diff --git a/.github/workflows/nix-ci.yml b/.github/workflows/nix-ci.yml index ac8b8c6ada7e..9c93570f6e8f 100644 --- a/.github/workflows/nix-ci.yml +++ b/.github/workflows/nix-ci.yml @@ -96,7 +96,7 @@ jobs: nix build $NIX_BUILD_ARGS .#cacheRoots -o push-build - name: Test run: | - nix build --keep-failed $NIX_BUILD_ARGS .#test -o push-test || (ln -s /tmp/nix-build-*/source/src/build/ ./push-test; false) + nix build --keep-failed $NIX_BUILD_ARGS .#test -o push-test || (ln -s /tmp/nix-build-*/build/source/src/build ./push-test; false) - name: Test Summary uses: test-summary/action@v2 with: diff --git a/doc/make/msys2.md b/doc/make/msys2.md index 2ec561f15526..2353449a9c7e 100644 --- a/doc/make/msys2.md +++ b/doc/make/msys2.md @@ -15,6 +15,13 @@ Mode](https://docs.microsoft.com/en-us/windows/apps/get-started/enable-your-devi which will allow Lean to create symlinks that e.g. enable go-to-definition in the stdlib. +## Installing the Windows SDK + +Install the Windows SDK from [Microsoft](https://developer.microsoft.com/en-us/windows/downloads/windows-sdk/). +The oldest supported version is 10.0.18362.0. If you installed the Windows SDK to the default location, +then there should be a directory with the version number at `C:\Program Files (x86)\Windows Kits\10\Include`. +If there are multiple directories, only the highest version number matters. + ## Installing dependencies [The official webpage of MSYS2][msys2] provides one-click installers. diff --git a/doc/monads/applicatives.lean b/doc/monads/applicatives.lean index dd19b081401c..3bf69c0260dd 100644 --- a/doc/monads/applicatives.lean +++ b/doc/monads/applicatives.lean @@ -138,8 +138,8 @@ definition: -/ instance : Applicative List where - pure := List.pure - seq f x := List.bind f fun y => Functor.map y (x ()) + pure := List.singleton + seq f x := List.flatMap f fun y => Functor.map y (x ()) /-! Notice you can now sequence a _list_ of functions and a _list_ of items. diff --git a/doc/monads/laws.lean b/doc/monads/laws.lean index bef495a1c3c8..d37c70b08185 100644 --- a/doc/monads/laws.lean +++ b/doc/monads/laws.lean @@ -128,8 +128,8 @@ Applying the identity function through an applicative structure should not chang values or structure. For example: -/ instance : Applicative List where - pure := List.pure - seq f x := List.bind f fun y => Functor.map y (x ()) + pure := List.singleton + seq f x := List.flatMap f fun y => Functor.map y (x ()) #eval pure id <*> [1, 2, 3] -- [1, 2, 3] /-! @@ -235,8 +235,8 @@ structure or its values. Left identity is `x >>= pure = x` and is demonstrated by the following examples on a monadic `List`: -/ instance : Monad List where - pure := List.pure - bind := List.bind + pure := List.singleton + bind := List.flatMap def a := ["apple", "orange"] diff --git a/doc/monads/monads.lean b/doc/monads/monads.lean index c8919709a616..f2a44685aad2 100644 --- a/doc/monads/monads.lean +++ b/doc/monads/monads.lean @@ -192,8 +192,8 @@ implementation of `pure` and `bind`. -/ instance : Monad List where - pure := List.pure - bind := List.bind + pure := List.singleton + bind := List.flatMap /-! Like you saw with the applicative `seq` operator, the `bind` operator applies the given function diff --git a/doc/setup.md b/doc/setup.md index 330dff5c86e5..28de3664f8e1 100644 --- a/doc/setup.md +++ b/doc/setup.md @@ -7,7 +7,7 @@ Platforms built & tested by our CI, available as binary releases via elan (see b * x86-64 Linux with glibc 2.27+ * x86-64 macOS 10.15+ * aarch64 (Apple Silicon) macOS 10.15+ -* x86-64 Windows 10+ +* x86-64 Windows 11 (any version), Windows 10 (version 1903 or higher), Windows Server 2022 ### Tier 2 diff --git a/script/prepare-llvm-mingw.sh b/script/prepare-llvm-mingw.sh index 4d32632197c0..f3e1b0a65a20 100644 --- a/script/prepare-llvm-mingw.sh +++ b/script/prepare-llvm-mingw.sh @@ -31,14 +31,20 @@ cp /clang64/lib/{crtbegin,crtend,crt2,dllcrt2}.o stage1/lib/ # runtime (cd llvm; cp --parents lib/clang/*/lib/*/libclang_rt.builtins* ../stage1) # further dependencies -cp /clang64/lib/lib{m,bcrypt,mingw32,moldname,mingwex,msvcrt,pthread,advapi32,shell32,user32,kernel32,ucrtbase,psapi,iphlpapi,userenv,ws2_32,dbghelp,ole32}.* /clang64/lib/libgmp.a /clang64/lib/libuv.a llvm/lib/lib{c++,c++abi,unwind}.a stage1/lib/ +# Note: even though we're linking against libraries like `libbcrypt.a` which appear to be static libraries from the file name, +# we're not actually linking statically against the code. +# Rather, `libbcrypt.a` is an import library (see https://en.wikipedia.org/wiki/Dynamic-link_library#Import_libraries) that just +# tells the compiler how to dynamically link against `bcrypt.dll` (which is located in the System32 folder). +# This distinction is relevant specifically for `libicu.a`/`icu.dll` because there we want updates to the time zone database to +# be delivered to users via Windows Update without having to recompile Lean or Lean programs. +cp /clang64/lib/lib{m,bcrypt,mingw32,moldname,mingwex,msvcrt,pthread,advapi32,shell32,user32,kernel32,ucrtbase,psapi,iphlpapi,userenv,ws2_32,dbghelp,ole32,icu}.* /clang64/lib/libgmp.a /clang64/lib/libuv.a llvm/lib/lib{c++,c++abi,unwind}.a stage1/lib/ echo -n " -DLEAN_STANDALONE=ON" echo -n " -DCMAKE_C_COMPILER=$PWD/stage1/bin/clang.exe -DCMAKE_C_COMPILER_WORKS=1 -DCMAKE_CXX_COMPILER=$PWD/llvm/bin/clang++.exe -DCMAKE_CXX_COMPILER_WORKS=1 -DLEAN_CXX_STDLIB='-lc++ -lc++abi'" echo -n " -DSTAGE0_CMAKE_C_COMPILER=clang -DSTAGE0_CMAKE_CXX_COMPILER=clang++" echo -n " -DLEAN_EXTRA_CXX_FLAGS='--sysroot $PWD/llvm -idirafter /clang64/include/'" echo -n " -DLEANC_INTERNAL_FLAGS='--sysroot ROOT -nostdinc -isystem ROOT/include/clang' -DLEANC_CC=ROOT/bin/clang.exe" echo -n " -DLEANC_INTERNAL_LINKER_FLAGS='-L ROOT/lib -static-libgcc -Wl,-Bstatic -lgmp $(pkg-config --static --libs libuv) -lunwind -Wl,-Bdynamic -fuse-ld=lld'" -# when not using the above flags, link GMP dynamically/as usual +# when not using the above flags, link GMP dynamically/as usual. Always link ICU dynamically. echo -n " -DLEAN_EXTRA_LINKER_FLAGS='-lgmp $(pkg-config --libs libuv) -lucrtbase'" # do not set `LEAN_CC` for tests echo -n " -DAUTO_THREAD_FINALIZATION=OFF -DSTAGE0_AUTO_THREAD_FINALIZATION=OFF" diff --git a/src/CMakeLists.txt b/src/CMakeLists.txt index 2b36ee213b2c..56b9bf8bd410 100644 --- a/src/CMakeLists.txt +++ b/src/CMakeLists.txt @@ -155,6 +155,10 @@ endif () # We want explicit stack probes in huge Lean stack frames for robust stack overflow detection string(APPEND LEANC_EXTRA_FLAGS " -fstack-clash-protection") +# This makes signed integer overflow guaranteed to match 2's complement. +string(APPEND CMAKE_CXX_FLAGS " -fwrapv") +string(APPEND LEANC_EXTRA_FLAGS " -fwrapv") + if(NOT MULTI_THREAD) message(STATUS "Disabled multi-thread support, it will not be safe to run multiple threads in parallel") set(AUTO_THREAD_FINALIZATION OFF) @@ -297,6 +301,23 @@ if(NOT LEAN_STANDALONE) string(APPEND LEAN_EXTRA_LINKER_FLAGS " ${LIBUV_LIBRARIES}") endif() +# Windows SDK (for ICU) +if(${CMAKE_SYSTEM_NAME} MATCHES "Windows") + # Pass 'tools' to skip MSVC version check (as MSVC/Visual Studio is not necessarily installed) + find_package(WindowsSDK REQUIRED COMPONENTS tools) + + # This will give a semicolon-separated list of include directories + get_windowssdk_include_dirs(${WINDOWSSDK_LATEST_DIR} WINDOWSSDK_INCLUDE_DIRS) + + # To successfully build against Windows SDK headers, the Windows SDK headers must have lower + # priority than other system headers, so use `-idirafter`. Unfortunately, CMake does not + # support this using `include_directories`. + string(REPLACE ";" "\" -idirafter \"" WINDOWSSDK_INCLUDE_DIRS "${WINDOWSSDK_INCLUDE_DIRS}") + string(APPEND CMAKE_CXX_FLAGS " -idirafter \"${WINDOWSSDK_INCLUDE_DIRS}\"") + + string(APPEND LEAN_EXTRA_LINKER_FLAGS " -licu") +endif() + # ccache if(CCACHE AND NOT CMAKE_CXX_COMPILER_LAUNCHER AND NOT CMAKE_C_COMPILER_LAUNCHER) find_program(CCACHE_PATH ccache) @@ -480,7 +501,7 @@ endif() # Git HASH if(USE_GITHASH) include(GetGitRevisionDescription) - get_git_head_revision(GIT_REFSPEC GIT_SHA1) + get_git_head_revision(GIT_REFSPEC GIT_SHA1 ALLOW_LOOKING_ABOVE_CMAKE_SOURCE_DIR) if(${GIT_SHA1} MATCHES "GITDIR-NOTFOUND") message(STATUS "Failed to read git_sha1") set(GIT_SHA1 "") diff --git a/src/Init/Control/Basic.lean b/src/Init/Control/Basic.lean index 61a73e9228c4..219130d1e1a9 100644 --- a/src/Init/Control/Basic.lean +++ b/src/Init/Control/Basic.lean @@ -8,6 +8,28 @@ import Init.Core universe u v w +/-- +A `ForIn'` instance, which handles `for h : x in c do`, +can also handle `for x in x do` by ignoring `h`, and so provides a `ForIn` instance. +-/ +instance (priority := low) instForInOfForIn' [ForIn' m ρ α d] : ForIn m ρ α where + forIn x b f := forIn' x b fun a _ => f a + +@[simp] theorem forIn'_eq_forIn [d : Membership α ρ] [ForIn' m ρ α d] {β} [Monad m] (x : ρ) (b : β) + (f : (a : α) → a ∈ x → β → m (ForInStep β)) (g : (a : α) → β → m (ForInStep β)) + (h : ∀ a m b, f a m b = g a b) : + forIn' x b f = forIn x b g := by + simp [instForInOfForIn'] + congr + apply funext + intro a + apply funext + intro m + apply funext + intro b + simp [h] + rfl + @[reducible] def Functor.mapRev {f : Type u → Type v} [Functor f] {α β : Type u} : f α → (α → β) → f β := fun a f => f <$> a diff --git a/src/Init/Control/StateRef.lean b/src/Init/Control/StateRef.lean index b4185766a11f..6aa41d8c273a 100644 --- a/src/Init/Control/StateRef.lean +++ b/src/Init/Control/StateRef.lean @@ -6,8 +6,7 @@ Authors: Leonardo de Moura, Sebastian Ullrich The State monad transformer using IO references. -/ prelude -import Init.System.IO -import Init.Control.State +import Init.System.ST def StateRefT' (ω : Type) (σ : Type) (m : Type → Type) (α : Type) : Type := ReaderT (ST.Ref ω σ) m α diff --git a/src/Init/Core.lean b/src/Init/Core.lean index b98fb6afdf40..46b3644d1961 100644 --- a/src/Init/Core.lean +++ b/src/Init/Core.lean @@ -324,7 +324,6 @@ class ForIn' (m : Type u₁ → Type u₂) (ρ : Type u) (α : outParam (Type v) export ForIn' (forIn') - /-- Auxiliary type used to compile `do` notation. It is used when compiling a do block nested inside a combinator like `tryCatch`. It encodes the possible ways the diff --git a/src/Init/Data.lean b/src/Init/Data.lean index 5034afda0e4d..87c642b95a22 100644 --- a/src/Init/Data.lean +++ b/src/Init/Data.lean @@ -19,6 +19,7 @@ import Init.Data.ByteArray import Init.Data.FloatArray import Init.Data.Fin import Init.Data.UInt +import Init.Data.SInt import Init.Data.Float import Init.Data.Option import Init.Data.Ord diff --git a/src/Init/Data/Array/Basic.lean b/src/Init/Data/Array/Basic.lean index 88117d0654b2..fec1b7bfee4c 100644 --- a/src/Init/Data/Array/Basic.lean +++ b/src/Init/Data/Array/Basic.lean @@ -82,6 +82,22 @@ theorem ext' {as bs : Array α} (h : as.toList = bs.toList) : as = bs := by @[simp] theorem getElem_toList {a : Array α} {i : Nat} (h : i < a.size) : a.toList[i] = a[i] := rfl +/-- `a ∈ as` is a predicate which asserts that `a` is in the array `as`. -/ +-- NB: This is defined as a structure rather than a plain def so that a lemma +-- like `sizeOf_lt_of_mem` will not apply with no actual arrays around. +structure Mem (as : Array α) (a : α) : Prop where + val : a ∈ as.toList + +instance : Membership α (Array α) where + mem := Mem + +theorem mem_def {a : α} {as : Array α} : a ∈ as ↔ a ∈ as.toList := + ⟨fun | .mk h => h, Array.Mem.mk⟩ + +@[simp] theorem getElem_mem {l : Array α} {i : Nat} (h : i < l.size) : l[i] ∈ l := by + rw [Array.mem_def, ← getElem_toList] + apply List.getElem_mem + end Array namespace List @@ -316,6 +332,37 @@ 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` -/ +@[inline] unsafe def forIn'Unsafe {α : Type u} {β : Type v} {m : Type v → Type w} [Monad m] (as : Array α) (b : β) (f : (a : α) → a ∈ as → β → m (ForInStep β)) : m β := + let sz := as.usize + let rec @[specialize] loop (i : USize) (b : β) : m β := do + if i < sz then + let a := as.uget i lcProof + match (← f a lcProof b) with + | ForInStep.done b => pure b + | ForInStep.yield b => loop (i+1) b + else + pure b + loop 0 b + +/-- Reference implementation for `forIn'` -/ +@[implemented_by Array.forIn'Unsafe] +protected def forIn' {α : Type u} {β : Type v} {m : Type v → Type w} [Monad m] (as : Array α) (b : β) (f : (a : α) → a ∈ as → β → m (ForInStep β)) : m β := + let rec loop (i : Nat) (h : i ≤ as.size) (b : β) : m β := do + match i, h with + | 0, _ => pure b + | i+1, h => + have h' : i < as.size := Nat.lt_of_lt_of_le (Nat.lt_succ_self i) h + have : as.size - 1 < as.size := Nat.sub_lt (Nat.zero_lt_of_lt h') (by decide) + have : as.size - 1 - i < as.size := Nat.lt_of_le_of_lt (Nat.sub_le (as.size - 1) i) this + match (← f as[as.size - 1 - i] (getElem_mem this) b) with + | ForInStep.done b => pure b + | ForInStep.yield b => loop i (Nat.le_of_lt h') b + loop as.size (Nat.le_refl _) b + +instance : ForIn' m (Array α) α inferInstance where + forIn' := Array.forIn' + /-- 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 β := diff --git a/src/Init/Data/Array/Lemmas.lean b/src/Init/Data/Array/Lemmas.lean index 2df2a3129179..474491cb3b3f 100644 --- a/src/Init/Data/Array/Lemmas.lean +++ b/src/Init/Data/Array/Lemmas.lean @@ -21,8 +21,7 @@ namespace Array @[simp] theorem getElem_mk {xs : List α} {i : Nat} (h : i < xs.length) : (Array.mk xs)[i] = xs[i] := rfl -theorem getElem_eq_getElem_toList {a : Array α} (h : i < a.size) : a[i] = a.toList[i] := by - by_cases i < a.size <;> (try simp [*]) <;> rfl +theorem getElem_eq_getElem_toList {a : Array α} (h : i < a.size) : a[i] = a.toList[i] := rfl theorem getElem?_eq_getElem {a : Array α} {i : Nat} (h : i < a.size) : a[i]? = some a[i] := getElem?_pos .. @@ -85,6 +84,9 @@ We prefer to pull `List.toArray` outwards. (a.toArrayAux b).size = b.size + a.length := by simp [size] +@[simp] theorem mem_toArray {a : α} {l : List α} : a ∈ l.toArray ↔ a ∈ l := by + simp [mem_def] + @[simp] theorem push_toArray (l : List α) (a : α) : l.toArray.push a = (l ++ [a]).toArray := by apply ext' simp @@ -121,6 +123,30 @@ We prefer to pull `List.toArray` outwards. rw [Array.forIn, forIn_loop_toArray] simp +@[simp] theorem forIn'_loop_toArray [Monad m] (l : List α) (f : (a : α) → a ∈ l.toArray → β → m (ForInStep β)) (i : Nat) + (h : i ≤ l.length) (b : β) : + Array.forIn'.loop l.toArray f i h b = + forIn' (l.drop (l.length - i)) b (fun a m b => f a (by simpa using mem_of_mem_drop m) b) := by + induction i generalizing l b with + | zero => + simp [Array.forIn'.loop] + | succ i ih => + simp only [Array.forIn'.loop, size_toArray, getElem_toArray, ih, forIn_eq_forIn] + have t : drop (l.length - (i + 1)) l = l[l.length - i - 1] :: drop (l.length - i) l := by + simp only [Nat.sub_add_eq] + rw [List.drop_sub_one (by omega), List.getElem?_eq_getElem (by omega)] + simp only [Option.toList_some, singleton_append] + simp [t] + have t : l.length - 1 - i = l.length - i - 1 := by omega + simp only [t] + congr + +@[simp] theorem forIn'_toArray [Monad m] (l : List α) (b : β) (f : (a : α) → a ∈ l.toArray → β → m (ForInStep β)) : + forIn' l.toArray b f = forIn' l b (fun a m b => f a (mem_toArray.mpr m) b) := by + change Array.forIn' _ _ _ = List.forIn' _ _ _ + rw [Array.forIn', forIn'_loop_toArray] + simp [List.forIn_eq_forIn] + theorem foldrM_toArray [Monad m] (f : α → β → m β) (init : β) (l : List α) : l.toArray.foldrM f init = l.foldrM f init := by rw [foldrM_eq_reverse_foldlM_toList] @@ -189,6 +215,9 @@ namespace Array @[simp] theorem size_mk (as : List α) : (Array.mk as).size = as.length := by simp [size] +@[simp] theorem isEmpty_toList {l : Array α} : l.toList.isEmpty = l.isEmpty := by + rcases l with ⟨_ | _⟩ <;> simp + theorem foldrM_push [Monad m] (f : α → β → m β) (init : β) (arr : Array α) (a : α) : (arr.push a).foldrM f init = f a init >>= arr.foldrM f := by simp [foldrM_eq_reverse_foldlM_toList, -size_push] @@ -265,9 +294,6 @@ theorem anyM_stop_le_start [Monad m] (p : α → m Bool) (as : Array α) (start (h : min stop as.size ≤ start) : anyM p as start stop = pure false := by rw [anyM_eq_anyM_loop, anyM.loop, dif_neg (Nat.not_lt.2 h)] -theorem mem_def {a : α} {as : Array α} : a ∈ as ↔ a ∈ as.toList := - ⟨fun | .mk h => h, Array.Mem.mk⟩ - @[simp] theorem not_mem_empty (a : α) : ¬(a ∈ #[]) := by simp [mem_def] @@ -457,10 +483,6 @@ theorem lt_of_getElem {x : α} {a : Array α} {idx : Nat} {hidx : idx < a.size} idx < a.size := hidx -@[simp] theorem getElem_mem {l : Array α} {i : Nat} (h : i < l.size) : l[i] ∈ l := by - erw [Array.mem_def, getElem_eq_getElem_toList] - apply List.get_mem - theorem getElem_fin_eq_getElem_toList (a : Array α) (i : Fin a.size) : a[i] = a.toList[i] := rfl @[simp] theorem ugetElem_eq_getElem (a : Array α) {i : USize} (h : i.toNat < a.size) : @@ -725,6 +747,11 @@ theorem getElem_range {n : Nat} {x : Nat} (h : x < (Array.range n).size) : (Arra cases as simp +@[simp] theorem forIn'_toList [Monad m] (as : Array α) (b : β) (f : (a : α) → a ∈ as.toList → β → m (ForInStep β)) : + forIn' as.toList b f = forIn' as b (fun a m b => f a (mem_toList.mpr m) b) := by + cases as + simp + /-! ### foldl / foldr -/ @[simp] theorem foldlM_loop_empty [Monad m] (f : β → α → m β) (init : β) (i j : Nat) : @@ -1018,18 +1045,38 @@ theorem getElem_append_right {as bs : Array α} {h : i < (as ++ bs).size} (hle : conv => rhs; rw [← List.getElem_append_right (h₁ := hle) (h₂ := h')] apply List.get_of_eq; rw [toList_append] +theorem getElem?_append_left {as bs : Array α} {n : Nat} (hn : n < as.size) : + (as ++ bs)[n]? = as[n]? := by + have hn' : n < (as ++ bs).size := Nat.lt_of_lt_of_le hn <| + size_append .. ▸ Nat.le_add_right .. + simp_all [getElem?_eq_getElem, getElem_append] + +theorem getElem?_append_right {as bs : Array α} {n : Nat} (h : as.size ≤ n) : + (as ++ bs)[n]? = bs[n - as.size]? := by + cases as + cases bs + simp at h + simp [List.getElem?_append_right, h] + +theorem getElem?_append {as bs : Array α} {n : Nat} : + (as ++ bs)[n]? = if n < as.size then as[n]? else bs[n - as.size]? := by + split <;> rename_i h + · exact getElem?_append_left h + · exact getElem?_append_right (by simpa using h) + @[simp] theorem append_nil (as : Array α) : as ++ #[] = as := by apply ext'; simp only [toList_append, toList_empty, List.append_nil] @[simp] theorem nil_append (as : Array α) : #[] ++ as = as := by apply ext'; simp only [toList_append, toList_empty, List.nil_append] -theorem append_assoc (as bs cs : Array α) : as ++ bs ++ cs = as ++ (bs ++ cs) := by +@[simp] theorem append_assoc (as bs cs : Array α) : as ++ bs ++ cs = as ++ (bs ++ cs) := by apply ext'; simp only [toList_append, List.append_assoc] /-! ### flatten -/ -@[simp] theorem toList_flatten {l : Array (Array α)} : l.flatten.toList = (l.toList.map toList).flatten := by +@[simp] theorem toList_flatten {l : Array (Array α)} : + l.flatten.toList = (l.toList.map toList).flatten := by dsimp [flatten] simp only [foldl_eq_foldl_toList] generalize l.toList = l @@ -1388,9 +1435,6 @@ namespace List Our goal is to have `simp` "pull `List.toArray` outwards" as much as possible. -/ -@[simp] theorem mem_toArray {a : α} {l : List α} : a ∈ l.toArray ↔ a ∈ l := by - simp [mem_def] - @[simp] theorem toListRev_toArray (l : List α) : l.toArray.toListRev = l.reverse := by simp diff --git a/src/Init/Data/Array/Mem.lean b/src/Init/Data/Array/Mem.lean index c33251ba3970..5887f4bb7fc9 100644 --- a/src/Init/Data/Array/Mem.lean +++ b/src/Init/Data/Array/Mem.lean @@ -10,15 +10,6 @@ import Init.Data.List.BasicAux namespace Array -/-- `a ∈ as` is a predicate which asserts that `a` is in the array `as`. -/ --- NB: This is defined as a structure rather than a plain def so that a lemma --- like `sizeOf_lt_of_mem` will not apply with no actual arrays around. -structure Mem (as : Array α) (a : α) : Prop where - val : a ∈ as.toList - -instance : Membership α (Array α) where - mem := Mem - theorem sizeOf_lt_of_mem [SizeOf α] {as : Array α} (h : a ∈ as) : sizeOf a < sizeOf as := by cases as with | _ as => exact Nat.lt_trans (List.sizeOf_lt_of_mem h.val) (by simp_arith) diff --git a/src/Init/Data/List/Basic.lean b/src/Init/Data/List/Basic.lean index 16146974629f..d9936e220c7a 100644 --- a/src/Init/Data/List/Basic.lean +++ b/src/Init/Data/List/Basic.lean @@ -29,7 +29,7 @@ The operations are organized as follow: * Lexicographic ordering: `lt`, `le`, and instances. * Head and tail operators: `head`, `head?`, `headD?`, `tail`, `tail?`, `tailD`. * Basic operations: - `map`, `filter`, `filterMap`, `foldr`, `append`, `flatten`, `pure`, `bind`, `replicate`, and + `map`, `filter`, `filterMap`, `foldr`, `append`, `flatten`, `pure`, `flatMap`, `replicate`, and `reverse`. * Additional functions defined in terms of these: `leftpad`, `rightPad`, and `reduceOption`. * Operations using indexes: `mapIdx`. diff --git a/src/Init/Data/List/Control.lean b/src/Init/Data/List/Control.lean index 7e6dc918c668..2f945829acd2 100644 --- a/src/Init/Data/List/Control.lean +++ b/src/Init/Data/List/Control.lean @@ -254,6 +254,8 @@ instance : ForIn m (List α) α where instance : ForIn' m (List α) α inferInstance where forIn' := List.forIn' +@[simp] theorem forIn'_eq_forIn' [Monad m] : @List.forIn' α β m _ = forIn' := rfl + @[simp] theorem forIn'_eq_forIn {α : Type u} {β : Type v} {m : Type v → Type w} [Monad m] (as : List α) (init : β) (f : α → β → m (ForInStep β)) : forIn' as init (fun a _ b => f a b) = forIn as init f := by simp [forIn', forIn, List.forIn, List.forIn'] have : ∀ cs h, List.forIn'.loop cs (fun a _ b => f a b) as init h = List.forIn.loop f as init := by diff --git a/src/Init/Data/List/Find.lean b/src/Init/Data/List/Find.lean index 90cd1369fe57..d493e0be5830 100644 --- a/src/Init/Data/List/Find.lean +++ b/src/Init/Data/List/Find.lean @@ -595,15 +595,14 @@ theorem findIdx_eq {p : α → Bool} {xs : List α} {i : Nat} (h : i < xs.length theorem findIdx_append (p : α → Bool) (l₁ l₂ : List α) : (l₁ ++ l₂).findIdx p = - if ∃ x, x ∈ l₁ ∧ p x = true then l₁.findIdx p else l₂.findIdx p + l₁.length := by + if l₁.findIdx p < l₁.length then l₁.findIdx p else l₂.findIdx p + l₁.length := by induction l₁ with | nil => simp | cons x xs ih => simp only [findIdx_cons, length_cons, cons_append] by_cases h : p x · simp [h] - · simp only [h, ih, cond_eq_if, Bool.false_eq_true, ↓reduceIte, mem_cons, exists_eq_or_imp, - false_or] + · simp only [h, ih, cond_eq_if, Bool.false_eq_true, ↓reduceIte, add_one_lt_add_one_iff] split <;> simp [Nat.add_assoc] theorem IsPrefix.findIdx_le {l₁ l₂ : List α} {p : α → Bool} (h : l₁ <+: l₂) : diff --git a/src/Init/Data/List/Lemmas.lean b/src/Init/Data/List/Lemmas.lean index b89341f4cc6b..1112ba8f650a 100644 --- a/src/Init/Data/List/Lemmas.lean +++ b/src/Init/Data/List/Lemmas.lean @@ -492,10 +492,6 @@ theorem getElem?_of_mem {a} {l : List α} (h : a ∈ l) : ∃ n : Nat, l[n]? = s theorem get?_of_mem {a} {l : List α} (h : a ∈ l) : ∃ n, l.get? n = some a := let ⟨⟨n, _⟩, e⟩ := get_of_mem h; ⟨n, e ▸ get?_eq_get _⟩ -@[simp] theorem getElem_mem : ∀ {l : List α} {n} (h : n < l.length), l[n]'h ∈ l - | _ :: _, 0, _ => .head .. - | _ :: l, _+1, _ => .tail _ (getElem_mem (l := l) ..) - theorem get_mem : ∀ (l : List α) n h, get l ⟨n, h⟩ ∈ l | _ :: _, 0, _ => .head .. | _ :: l, _+1, _ => .tail _ (get_mem l ..) diff --git a/src/Init/Data/List/Monadic.lean b/src/Init/Data/List/Monadic.lean index 04dcfda7d858..f8ded7d6f284 100644 --- a/src/Init/Data/List/Monadic.lean +++ b/src/Init/Data/List/Monadic.lean @@ -87,6 +87,68 @@ theorem mapM_eq_reverse_foldlM_cons [Monad m] [LawfulMonad m] (f : α → m β) (l₁ ++ l₂).forM f = (do l₁.forM f; l₂.forM f) := by induction l₁ <;> simp [*] +/-! ### forIn' -/ + +@[simp] theorem forIn'_nil [Monad m] (f : (a : α) → a ∈ [] → β → m (ForInStep β)) (b : β) : forIn' [] b f = pure b := + rfl + +theorem forIn'_loop_congr [Monad m] {as bs : List α} + {f : (a' : α) → a' ∈ as → β → m (ForInStep β)} + {g : (a' : α) → a' ∈ bs → β → m (ForInStep β)} + {b : β} (ha : ∃ ys, ys ++ xs = as) (hb : ∃ ys, ys ++ xs = bs) + (h : ∀ a m m' b, f a m b = g a m' b) : forIn'.loop as f xs b ha = forIn'.loop bs g xs b hb := by + induction xs generalizing b with + | nil => simp [forIn'.loop] + | cons a xs ih => + simp only [forIn'.loop] at * + congr 1 + · rw [h] + · funext s + obtain b | b := s + · rfl + · simp + rw [ih] + +@[simp] theorem forIn'_cons [Monad m] {a : α} {as : List α} + (f : (a' : α) → a' ∈ a :: as → β → m (ForInStep β)) (b : β) : + forIn' (a::as) b f = f a (mem_cons_self a as) b >>= + fun | ForInStep.done b => pure b | ForInStep.yield b => forIn' as b fun a' m b => f a' (mem_cons_of_mem a m) b := by + simp only [forIn', List.forIn', forIn'.loop] + congr 1 + funext s + obtain b | b := s + · rfl + · apply forIn'_loop_congr + intros + rfl + +@[congr] theorem forIn'_congr [Monad m] {as bs : List α} (w : as = bs) + {b b' : β} (hb : b = b') + {f : (a' : α) → a' ∈ as → β → m (ForInStep β)} + {g : (a' : α) → a' ∈ bs → β → m (ForInStep β)} + (h : ∀ a m b, f a (by simpa [w] using m) b = g a m b) : + forIn' as b f = forIn' bs b' g := by + induction bs generalizing as b b' with + | nil => + subst w + simp [hb, forIn'_nil] + | cons b bs ih => + cases as with + | nil => simp at w + | cons a as => + simp only [cons.injEq] at w + obtain ⟨rfl, rfl⟩ := w + simp only [forIn'_cons] + congr 1 + · simp [h, hb] + · funext s + obtain b | b := s + · rfl + · simp + rw [ih rfl rfl] + intro a m b + exact h a (mem_cons_of_mem _ m) b + /-! ### allM -/ theorem allM_eq_not_anyM_not [Monad m] [LawfulMonad m] (p : α → m Bool) (as : List α) : diff --git a/src/Init/Data/List/Nat/Modify.lean b/src/Init/Data/List/Nat/Modify.lean index 6fdff06f60d0..c1a112e9fe7f 100644 --- a/src/Init/Data/List/Nat/Modify.lean +++ b/src/Init/Data/List/Nat/Modify.lean @@ -6,25 +6,79 @@ Authors: Parikshit Khanna, Jeremy Avigad, Leonardo de Moura, Floris van Doorn, M prelude import Init.Data.List.Nat.TakeDrop +import Init.Data.List.Nat.Erase namespace List /-! ### modifyHead -/ -@[simp] theorem modifyHead_modifyHead (l : List α) (f g : α → α) : +@[simp] theorem length_modifyHead {f : α → α} {l : List α} : (l.modifyHead f).length = l.length := by + cases l <;> simp [modifyHead] + +theorem modifyHead_eq_set [Inhabited α] (f : α → α) (l : List α) : + l.modifyHead f = l.set 0 (f (l[0]?.getD default)) := by cases l <;> simp [modifyHead] + +@[simp] theorem modifyHead_eq_nil_iff {f : α → α} {l : List α} : + l.modifyHead f = [] ↔ l = [] := by cases l <;> simp [modifyHead] + +@[simp] theorem modifyHead_modifyHead {l : List α} {f g : α → α} : (l.modifyHead f).modifyHead g = l.modifyHead (g ∘ f) := by cases l <;> simp [modifyHead] -/-! ### modify -/ +theorem getElem_modifyHead {l : List α} {f : α → α} {n} (h : n < (l.modifyHead f).length) : + (l.modifyHead f)[n] = if h' : n = 0 then f (l[0]'(by simp at h; omega)) else l[n]'(by simpa using h) := by + cases l with + | nil => simp at h + | cons hd tl => cases n <;> simp -@[simp] theorem modify_nil (f : α → α) (n) : [].modify f n = [] := by cases n <;> rfl +@[simp] theorem getElem_modifyHead_zero {l : List α} {f : α → α} {h} : + (l.modifyHead f)[0] = f (l[0]'(by simpa using h)) := by simp [getElem_modifyHead] -@[simp] theorem modify_zero_cons (f : α → α) (a : α) (l : List α) : - (a :: l).modify f 0 = f a :: l := rfl +@[simp] theorem getElem_modifyHead_succ {l : List α} {f : α → α} {n} (h : n + 1 < (l.modifyHead f).length) : + (l.modifyHead f)[n + 1] = l[n + 1]'(by simpa using h) := by simp [getElem_modifyHead] -@[simp] theorem modify_succ_cons (f : α → α) (a : α) (l : List α) (n) : - (a :: l).modify f (n + 1) = a :: l.modify f n := by rfl +theorem getElem?_modifyHead {l : List α} {f : α → α} {n} : + (l.modifyHead f)[n]? = if n = 0 then l[n]?.map f else l[n]? := by + cases l with + | nil => simp + | cons hd tl => cases n <;> simp + +@[simp] theorem getElem?_modifyHead_zero {l : List α} {f : α → α} : + (l.modifyHead f)[0]? = l[0]?.map f := by simp [getElem?_modifyHead] + +@[simp] theorem getElem?_modifyHead_succ {l : List α} {f : α → α} {n} : + (l.modifyHead f)[n + 1]? = l[n + 1]? := by simp [getElem?_modifyHead] + +@[simp] theorem head_modifyHead (f : α → α) (l : List α) (h) : + (l.modifyHead f).head h = f (l.head (by simpa using h)) := by + cases l with + | nil => simp at h + | cons hd tl => simp -theorem modifyTailIdx_id : ∀ n (l : List α), l.modifyTailIdx id n = l +@[simp] theorem head?_modifyHead {l : List α} {f : α → α} : + (l.modifyHead f).head? = l.head?.map f := by cases l <;> simp + +@[simp] theorem tail_modifyHead {f : α → α} {l : List α} : + (l.modifyHead f).tail = l.tail := by cases l <;> simp + +@[simp] theorem take_modifyHead {f : α → α} {l : List α} {n} : + (l.modifyHead f).take n = (l.take n).modifyHead f := by + cases l <;> cases n <;> simp + +@[simp] theorem drop_modifyHead_of_pos {f : α → α} {l : List α} {n} (h : 0 < n) : + (l.modifyHead f).drop n = l.drop n := by + cases l <;> cases n <;> simp_all + +@[simp] theorem eraseIdx_modifyHead_zero {f : α → α} {l : List α} : + (l.modifyHead f).eraseIdx 0 = l.eraseIdx 0 := by cases l <;> simp + +@[simp] theorem eraseIdx_modifyHead_of_pos {f : α → α} {l : List α} {n} (h : 0 < n) : + (l.modifyHead f).eraseIdx n = (l.eraseIdx n).modifyHead f := by cases l <;> cases n <;> simp_all + +@[simp] theorem modifyHead_id : modifyHead (id : α → α) = id := by funext l; cases l <;> simp + +/-! ### modifyTailIdx -/ + +@[simp] theorem modifyTailIdx_id : ∀ n (l : List α), l.modifyTailIdx id n = l | 0, _ => rfl | _+1, [] => rfl | n+1, a :: l => congrArg (cons a) (modifyTailIdx_id n l) @@ -34,6 +88,44 @@ theorem eraseIdx_eq_modifyTailIdx : ∀ n (l : List α), eraseIdx l n = modifyTa | _+1, [] => rfl | _+1, _ :: _ => congrArg (cons _) (eraseIdx_eq_modifyTailIdx _ _) +@[simp] theorem length_modifyTailIdx (f : List α → List α) (H : ∀ l, length (f l) = length l) : + ∀ n l, length (modifyTailIdx f n l) = length l + | 0, _ => H _ + | _+1, [] => rfl + | _+1, _ :: _ => congrArg (·+1) (length_modifyTailIdx _ H _ _) + +theorem modifyTailIdx_add (f : List α → List α) (n) (l₁ l₂ : List α) : + modifyTailIdx f (l₁.length + n) (l₁ ++ l₂) = l₁ ++ modifyTailIdx f n l₂ := by + induction l₁ <;> simp [*, Nat.succ_add] + +theorem modifyTailIdx_eq_take_drop (f : List α → List α) (H : f [] = []) : + ∀ n l, modifyTailIdx f n l = take n l ++ f (drop n l) + | 0, _ => rfl + | _ + 1, [] => H.symm + | n + 1, b :: l => congrArg (cons b) (modifyTailIdx_eq_take_drop f H n l) + +theorem exists_of_modifyTailIdx (f : List α → List α) {n} {l : List α} (h : n ≤ l.length) : + ∃ l₁ l₂, l = l₁ ++ l₂ ∧ l₁.length = n ∧ modifyTailIdx f n l = l₁ ++ f l₂ := + have ⟨_, _, eq, hl⟩ : ∃ l₁ l₂, l = l₁ ++ l₂ ∧ l₁.length = n := + ⟨_, _, (take_append_drop n l).symm, length_take_of_le h⟩ + ⟨_, _, eq, hl, hl ▸ eq ▸ modifyTailIdx_add (n := 0) ..⟩ + +/-! ### modify -/ + +@[simp] theorem modify_nil (f : α → α) (n) : [].modify f n = [] := by cases n <;> rfl + +@[simp] theorem modify_zero_cons (f : α → α) (a : α) (l : List α) : + (a :: l).modify f 0 = f a :: l := rfl + +@[simp] theorem modify_succ_cons (f : α → α) (a : α) (l : List α) (n) : + (a :: l).modify f (n + 1) = a :: l.modify f n := by rfl + +theorem modifyHead_eq_modify_zero (f : α → α) (l : List α) : + l.modifyHead f = l.modify f 0 := by cases l <;> simp + +@[simp] theorem modify_eq_nil_iff (f : α → α) (n) (l : List α) : + l.modify f n = [] ↔ l = [] := by cases l <;> cases n <;> simp + theorem getElem?_modify (f : α → α) : ∀ n (l : List α) m, (modify f n l)[m]? = (fun a => if n = m then f a else a) <$> l[m]? | n, l, 0 => by cases l <;> cases n <;> simp @@ -45,16 +137,6 @@ theorem getElem?_modify (f : α → α) : cases h' : l[m]? <;> by_cases h : n = m <;> simp [h, if_pos, if_neg, Option.map, mt Nat.succ.inj, not_false_iff, h'] -@[simp] theorem length_modifyTailIdx (f : List α → List α) (H : ∀ l, length (f l) = length l) : - ∀ n l, length (modifyTailIdx f n l) = length l - | 0, _ => H _ - | _+1, [] => rfl - | _+1, _ :: _ => congrArg (·+1) (length_modifyTailIdx _ H _ _) - -theorem modifyTailIdx_add (f : List α → List α) (n) (l₁ l₂ : List α) : - modifyTailIdx f (l₁.length + n) (l₁ ++ l₂) = l₁ ++ modifyTailIdx f n l₂ := by - induction l₁ <;> simp [*, Nat.succ_add] - @[simp] theorem length_modify (f : α → α) : ∀ n l, length (modify f n l) = length l := length_modifyTailIdx _ fun l => by cases l <;> rfl @@ -73,30 +155,141 @@ theorem getElem_modify (f : α → α) (n) (l : List α) (m) (h : m < (modify f simp at h simp [h] -theorem modifyTailIdx_eq_take_drop (f : List α → List α) (H : f [] = []) : - ∀ n l, modifyTailIdx f n l = take n l ++ f (drop n l) - | 0, _ => rfl - | _ + 1, [] => H.symm - | n + 1, b :: l => congrArg (cons b) (modifyTailIdx_eq_take_drop f H n l) +@[simp] theorem getElem_modify_eq (f : α → α) (n) (l : List α) (h) : + (modify f n l)[n] = f (l[n]'(by simpa using h)) := by simp [getElem_modify] + +@[simp] theorem getElem_modify_ne (f : α → α) {m n} (l : List α) (h : m ≠ n) (h') : + (modify f m l)[n] = l[n]'(by simpa using h') := by simp [getElem_modify, h] + +theorem modify_eq_self {f : α → α} {n} {l : List α} (h : l.length ≤ n) : + l.modify f n = l := by + apply ext_getElem + · simp + · intro m h₁ h₂ + simp only [getElem_modify, ite_eq_right_iff] + intro h + omega + +theorem modify_modify_eq (f g : α → α) (n) (l : List α) : + (modify f n l).modify g n = modify (g ∘ f) n l := by + apply ext_getElem + · simp + · intro m h₁ h₂ + simp only [getElem_modify, Function.comp_apply] + split <;> simp + +theorem modify_modify_ne (f g : α → α) {m n} (l : List α) (h : m ≠ n) : + (modify f m l).modify g n = (l.modify g n).modify f m := by + apply ext_getElem + · simp + · intro m' h₁ h₂ + simp only [getElem_modify, getElem_modify_ne, h₂] + split <;> split <;> first | rfl | omega + +theorem modify_eq_set [Inhabited α] (f : α → α) (n) (l : List α) : + modify f n l = l.set n (f (l[n]?.getD default)) := by + apply ext_getElem + · simp + · intro m h₁ h₂ + simp [getElem_modify, getElem_set, h₂] + split <;> rename_i h + · subst h + simp only [length_modify] at h₁ + simp [h₁] + · rfl theorem modify_eq_take_drop (f : α → α) : ∀ n l, modify f n l = take n l ++ modifyHead f (drop n l) := modifyTailIdx_eq_take_drop _ rfl -theorem modify_eq_take_cons_drop (f : α → α) {n l} (h : n < length l) : +theorem modify_eq_take_cons_drop {f : α → α} {n} {l : List α} (h : n < l.length) : modify f n l = take n l ++ f l[n] :: drop (n + 1) l := by rw [modify_eq_take_drop, drop_eq_getElem_cons h]; rfl -theorem exists_of_modifyTailIdx (f : List α → List α) {n} {l : List α} (h : n ≤ l.length) : - ∃ l₁ l₂, l = l₁ ++ l₂ ∧ l₁.length = n ∧ modifyTailIdx f n l = l₁ ++ f l₂ := - have ⟨_, _, eq, hl⟩ : ∃ l₁ l₂, l = l₁ ++ l₂ ∧ l₁.length = n := - ⟨_, _, (take_append_drop n l).symm, length_take_of_le h⟩ - ⟨_, _, eq, hl, hl ▸ eq ▸ modifyTailIdx_add (n := 0) ..⟩ - theorem exists_of_modify (f : α → α) {n} {l : List α} (h : n < l.length) : ∃ l₁ a l₂, l = l₁ ++ a :: l₂ ∧ l₁.length = n ∧ modify f n l = l₁ ++ f a :: l₂ := match exists_of_modifyTailIdx _ (Nat.le_of_lt h) with | ⟨_, _::_, eq, hl, H⟩ => ⟨_, _, _, eq, hl, H⟩ | ⟨_, [], eq, hl, _⟩ => nomatch Nat.ne_of_gt h (eq ▸ append_nil _ ▸ hl) +@[simp] theorem modify_id (n) (l : List α) : l.modify id n = l := by + simp [modify] + +theorem take_modify (f : α → α) (n m) (l : List α) : + (modify f m l).take n = (take n l).modify f m := by + induction n generalizing l m with + | zero => simp + | succ n ih => + cases l with + | nil => simp + | cons hd tl => + cases m with + | zero => simp + | succ m => simp [ih] + +theorem drop_modify_of_lt (f : α → α) (n m) (l : List α) (h : n < m) : + (modify f n l).drop m = l.drop m := by + apply ext_getElem + · simp + · intro m' h₁ h₂ + simp only [getElem_drop, getElem_modify, ite_eq_right_iff] + intro h' + omega + +theorem drop_modify_of_ge (f : α → α) (n m) (l : List α) (h : n ≥ m) : + (modify f n l).drop m = modify f (n - m) (drop m l) := by + apply ext_getElem + · simp + · intro m' h₁ h₂ + simp [getElem_drop, getElem_modify, ite_eq_right_iff] + split <;> split <;> first | rfl | omega + +theorem eraseIdx_modify_of_eq (f : α → α) (n) (l : List α) : + (modify f n l).eraseIdx n = l.eraseIdx n := by + apply ext_getElem + · simp [length_eraseIdx] + · intro m h₁ h₂ + simp only [getElem_eraseIdx, getElem_modify] + split <;> split <;> first | rfl | omega + +theorem eraseIdx_modify_of_lt (f : α → α) (i j) (l : List α) (h : j < i) : + (modify f i l).eraseIdx j = (l.eraseIdx j).modify f (i - 1) := by + apply ext_getElem + · simp [length_eraseIdx] + · intro k h₁ h₂ + simp only [getElem_eraseIdx, getElem_modify] + by_cases h' : i - 1 = k + repeat' split + all_goals (first | rfl | omega) + +theorem eraseIdx_modify_of_gt (f : α → α) (i j) (l : List α) (h : j > i) : + (modify f i l).eraseIdx j = (l.eraseIdx j).modify f i := by + apply ext_getElem + · simp [length_eraseIdx] + · intro k h₁ h₂ + simp only [getElem_eraseIdx, getElem_modify] + by_cases h' : i = k + repeat' split + all_goals (first | rfl | omega) + +theorem modify_eraseIdx_of_lt (f : α → α) (i j) (l : List α) (h : j < i) : + (l.eraseIdx i).modify f j = (l.modify f j).eraseIdx i := by + apply ext_getElem + · simp [length_eraseIdx] + · intro k h₁ h₂ + simp only [getElem_eraseIdx, getElem_modify] + by_cases h' : j = k + 1 + repeat' split + all_goals (first | rfl | omega) + +theorem modify_eraseIdx_of_ge (f : α → α) (i j) (l : List α) (h : j ≥ i) : + (l.eraseIdx i).modify f j = (l.modify f (j + 1)).eraseIdx i := by + apply ext_getElem + · simp [length_eraseIdx] + · intro k h₁ h₂ + simp only [getElem_eraseIdx, getElem_modify] + by_cases h' : j + 1 = k + 1 + repeat' split + all_goals (first | rfl | omega) + end List diff --git a/src/Init/Data/Option/Basic.lean b/src/Init/Data/Option/Basic.lean index 73a7d574bae6..a4ee792f62c7 100644 --- a/src/Init/Data/Option/Basic.lean +++ b/src/Init/Data/Option/Basic.lean @@ -4,9 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE. Authors: Leonardo de Moura, Mario Carneiro -/ prelude -import Init.Core import Init.Control.Basic -import Init.Coe namespace Option diff --git a/src/Init/Data/Option/List.lean b/src/Init/Data/Option/List.lean index aa22d3912d04..794e9f1e9d67 100644 --- a/src/Init/Data/Option/List.lean +++ b/src/Init/Data/Option/List.lean @@ -11,4 +11,28 @@ namespace Option @[simp] theorem mem_toList {a : α} {o : Option α} : a ∈ o.toList ↔ a ∈ o := by cases o <;> simp [eq_comm] +@[simp] theorem forIn'_none [Monad m] (b : β) (f : (a : α) → a ∈ none → β → m (ForInStep β)) : + forIn' none b f = pure b := by + rfl + +@[simp] theorem forIn'_some [Monad m] (a : α) (b : β) (f : (a' : α) → a' ∈ some a → β → m (ForInStep β)) : + forIn' (some a) b f = bind (f a rfl b) (fun | .done r | .yield r => pure r) := by + rfl + +@[simp] theorem forIn_none [Monad m] (b : β) (f : α → β → m (ForInStep β)) : + forIn none b f = pure b := by + rfl + +@[simp] theorem forIn_some [Monad m] (a : α) (b : β) (f : α → β → m (ForInStep β)) : + forIn (some a) b f = bind (f a b) (fun | .done r | .yield r => pure r) := by + rfl + +@[simp] theorem forIn'_toList [Monad m] (o : Option α) (b : β) (f : (a : α) → a ∈ o.toList → β → m (ForInStep β)) : + forIn' o.toList b f = forIn' o b fun a m b => f a (by simpa using m) b := by + cases o <;> rfl + +@[simp] theorem forIn_toList [Monad m] (o : Option α) (b : β) (f : α → β → m (ForInStep β)) : + forIn o.toList b f = forIn o b f := by + cases o <;> rfl + end Option diff --git a/src/Init/Data/Repr.lean b/src/Init/Data/Repr.lean index 9b363da289e1..50123a9ac6bb 100644 --- a/src/Init/Data/Repr.lean +++ b/src/Init/Data/Repr.lean @@ -5,10 +5,6 @@ Author: Leonardo de Moura -/ prelude import Init.Data.Format.Basic -import Init.Data.Int.Basic -import Init.Data.Nat.Div -import Init.Data.UInt.BasicAux -import Init.Control.Id open Sum Subtype Nat open Std diff --git a/src/Init/Data/SInt.lean b/src/Init/Data/SInt.lean new file mode 100644 index 000000000000..efbeb970b55b --- /dev/null +++ b/src/Init/Data/SInt.lean @@ -0,0 +1,11 @@ +/- +Copyright (c) 2024 Lean FRO, LLC. All rights reserved. +Released under Apache 2.0 license as described in the file LICENSE. +Authors: Henrik Böving +-/ +prelude +import Init.Data.SInt.Basic + +/-! +This module contains the definitions and basic theory about signed fixed width integer types. +-/ diff --git a/src/Init/Data/SInt/Basic.lean b/src/Init/Data/SInt/Basic.lean new file mode 100644 index 000000000000..55cdc761eb9f --- /dev/null +++ b/src/Init/Data/SInt/Basic.lean @@ -0,0 +1,116 @@ +/- +Copyright (c) 2024 Lean FRO, LLC. All rights reserved. +Released under Apache 2.0 license as described in the file LICENSE. +Authors: Henrik Böving +-/ +prelude +import Init.Data.UInt.Basic + +/-! +This module contains the definition of signed fixed width integer types as well as basic arithmetic +and bitwise operations on top of it. +-/ + + +/-- +The type of signed 8-bit integers. This type has special support in the +compiler to make it actually 8 bits rather than wrapping a `Nat`. +-/ +structure Int8 where + /-- + Obtain the `UInt8` that is 2's complement equivalent to the `Int8`. + -/ + toUInt8 : UInt8 + +/-- The size of type `Int8`, that is, `2^8 = 256`. -/ +abbrev Int8.size : Nat := 256 + +/-- +Obtain the `BitVec` that contains the 2's complement representation of the `Int8`. +-/ +@[inline] def Int8.toBitVec (x : Int8) : BitVec 8 := x.toUInt8.toBitVec + +@[extern "lean_int8_of_int"] +def Int8.ofInt (i : @& Int) : Int8 := ⟨⟨BitVec.ofInt 8 i⟩⟩ +@[extern "lean_int8_of_int"] +def Int8.ofNat (n : @& Nat) : Int8 := ⟨⟨BitVec.ofNat 8 n⟩⟩ +abbrev Int.toInt8 := Int8.ofInt +abbrev Nat.toInt8 := Int8.ofNat +@[extern "lean_int8_to_int"] +def Int8.toInt (i : Int8) : Int := i.toBitVec.toInt +@[inline] def Int8.toNat (i : Int8) : Nat := i.toInt.toNat +@[extern "lean_int8_neg"] +def Int8.neg (i : Int8) : Int8 := ⟨⟨-i.toBitVec⟩⟩ + +instance : ToString Int8 where + toString i := toString i.toInt + +instance : OfNat Int8 n := ⟨Int8.ofNat n⟩ +instance : Neg Int8 where + neg := Int8.neg + +@[extern "lean_int8_add"] +def Int8.add (a b : Int8) : Int8 := ⟨⟨a.toBitVec + b.toBitVec⟩⟩ +@[extern "lean_int8_sub"] +def Int8.sub (a b : Int8) : Int8 := ⟨⟨a.toBitVec - b.toBitVec⟩⟩ +@[extern "lean_int8_mul"] +def Int8.mul (a b : Int8) : Int8 := ⟨⟨a.toBitVec * b.toBitVec⟩⟩ +@[extern "lean_int8_div"] +def Int8.div (a b : Int8) : Int8 := ⟨⟨BitVec.sdiv a.toBitVec b.toBitVec⟩⟩ +@[extern "lean_int8_mod"] +def Int8.mod (a b : Int8) : Int8 := ⟨⟨BitVec.smod a.toBitVec b.toBitVec⟩⟩ +@[extern "lean_int8_land"] +def Int8.land (a b : Int8) : Int8 := ⟨⟨a.toBitVec &&& b.toBitVec⟩⟩ +@[extern "lean_int8_lor"] +def Int8.lor (a b : Int8) : Int8 := ⟨⟨a.toBitVec ||| b.toBitVec⟩⟩ +@[extern "lean_int8_xor"] +def Int8.xor (a b : Int8) : Int8 := ⟨⟨a.toBitVec ^^^ b.toBitVec⟩⟩ +@[extern "lean_int8_shift_left"] +def Int8.shiftLeft (a b : Int8) : Int8 := ⟨⟨a.toBitVec <<< (mod b 8).toBitVec⟩⟩ +@[extern "lean_int8_shift_right"] +def Int8.shiftRight (a b : Int8) : Int8 := ⟨⟨BitVec.sshiftRight' a.toBitVec (mod b 8).toBitVec⟩⟩ +@[extern "lean_int8_complement"] +def Int8.complement (a : Int8) : Int8 := ⟨⟨~~~a.toBitVec⟩⟩ + +@[extern "lean_int8_dec_eq"] +def Int8.decEq (a b : Int8) : Decidable (a = b) := + match a, b with + | ⟨n⟩, ⟨m⟩ => + if h : n = m then + isTrue <| h ▸ rfl + else + isFalse (fun h' => Int8.noConfusion h' (fun h' => absurd h' h)) + +def Int8.lt (a b : Int8) : Prop := a.toBitVec.slt b.toBitVec +def Int8.le (a b : Int8) : Prop := a.toBitVec.sle b.toBitVec + +instance : Inhabited Int8 where + default := 0 + +instance : Add Int8 := ⟨Int8.add⟩ +instance : Sub Int8 := ⟨Int8.sub⟩ +instance : Mul Int8 := ⟨Int8.mul⟩ +instance : Mod Int8 := ⟨Int8.mod⟩ +instance : Div Int8 := ⟨Int8.div⟩ +instance : LT Int8 := ⟨Int8.lt⟩ +instance : LE Int8 := ⟨Int8.le⟩ +instance : Complement Int8 := ⟨Int8.complement⟩ +instance : AndOp Int8 := ⟨Int8.land⟩ +instance : OrOp Int8 := ⟨Int8.lor⟩ +instance : Xor Int8 := ⟨Int8.xor⟩ +instance : ShiftLeft Int8 := ⟨Int8.shiftLeft⟩ +instance : ShiftRight Int8 := ⟨Int8.shiftRight⟩ +instance : DecidableEq Int8 := Int8.decEq + +@[extern "lean_int8_dec_lt"] +def Int8.decLt (a b : Int8) : Decidable (a < b) := + inferInstanceAs (Decidable (a.toBitVec.slt b.toBitVec)) + +@[extern "lean_int8_dec_le"] +def Int8.decLe (a b : Int8) : Decidable (a ≤ b) := + inferInstanceAs (Decidable (a.toBitVec.sle b.toBitVec)) + +instance (a b : Int8) : Decidable (a < b) := Int8.decLt a b +instance (a b : Int8) : Decidable (a ≤ b) := Int8.decLe a b +instance : Max Int8 := maxOfLe +instance : Min Int8 := minOfLe diff --git a/src/Init/Data/String/Basic.lean b/src/Init/Data/String/Basic.lean index 95fffe785c87..6851c3ef1334 100644 --- a/src/Init/Data/String/Basic.lean +++ b/src/Init/Data/String/Basic.lean @@ -6,7 +6,6 @@ Author: Leonardo de Moura, Mario Carneiro prelude import Init.Data.List.Basic import Init.Data.Char.Basic -import Init.Data.Option.Basic universe u diff --git a/src/Init/Data/ToString/Basic.lean b/src/Init/Data/ToString/Basic.lean index 06b3d85ff09b..57e777bf3301 100644 --- a/src/Init/Data/ToString/Basic.lean +++ b/src/Init/Data/ToString/Basic.lean @@ -4,14 +4,9 @@ Released under Apache 2.0 license as described in the file LICENSE. Author: Leonardo de Moura -/ prelude -import Init.Data.String.Basic -import Init.Data.UInt.BasicAux -import Init.Data.Nat.Div import Init.Data.Repr -import Init.Data.Int.Basic -import Init.Data.Format.Basic -import Init.Control.Id -import Init.Control.Option +import Init.Data.Option.Basic + open Sum Subtype Nat open Std diff --git a/src/Init/GetElem.lean b/src/Init/GetElem.lean index fc4b06040254..2906fd3204ea 100644 --- a/src/Init/GetElem.lean +++ b/src/Init/GetElem.lean @@ -144,22 +144,26 @@ instance (priority := low) [GetElem coll idx elem valid] [∀ xs i, Decidable (v LawfulGetElem coll idx elem valid where theorem getElem?_pos [GetElem? cont idx elem dom] [LawfulGetElem cont idx elem dom] - (c : cont) (i : idx) (h : dom c i) [Decidable (dom c i)] : c[i]? = some (c[i]'h) := by + (c : cont) (i : idx) (h : dom c i) : c[i]? = some (c[i]'h) := by + have : Decidable (dom c i) := .isTrue h rw [getElem?_def] exact dif_pos h theorem getElem?_neg [GetElem? cont idx elem dom] [LawfulGetElem cont idx elem dom] - (c : cont) (i : idx) (h : ¬dom c i) [Decidable (dom c i)] : c[i]? = none := by + (c : cont) (i : idx) (h : ¬dom c i) : c[i]? = none := by + have : Decidable (dom c i) := .isFalse h rw [getElem?_def] exact dif_neg h theorem getElem!_pos [GetElem? cont idx elem dom] [LawfulGetElem cont idx elem dom] - [Inhabited elem] (c : cont) (i : idx) (h : dom c i) [Decidable (dom c i)] : + [Inhabited elem] (c : cont) (i : idx) (h : dom c i) : c[i]! = c[i]'h := by + have : Decidable (dom c i) := .isTrue h simp [getElem!_def, getElem?_def, h] theorem getElem!_neg [GetElem? cont idx elem dom] [LawfulGetElem cont idx elem dom] - [Inhabited elem] (c : cont) (i : idx) (h : ¬dom c i) [Decidable (dom c i)] : c[i]! = default := by + [Inhabited elem] (c : cont) (i : idx) (h : ¬dom c i) : c[i]! = default := by + have : Decidable (dom c i) := .isFalse h simp [getElem!_def, getElem?_def, h] namespace Fin @@ -203,6 +207,10 @@ instance : GetElem (List α) Nat α fun as i => i < as.length where @[deprecated (since := "2024-06-12")] abbrev cons_getElem_succ := @getElem_cons_succ +@[simp] theorem getElem_mem : ∀ {l : List α} {n} (h : n < l.length), l[n]'h ∈ l + | _ :: _, 0, _ => .head .. + | _ :: l, _+1, _ => .tail _ (getElem_mem (l := l) ..) + theorem get_drop_eq_drop (as : List α) (i : Nat) (h : i < as.length) : as[i] :: as.drop (i+1) = as.drop i := match as, i with | _::_, 0 => rfl diff --git a/src/Init/System/FilePath.lean b/src/Init/System/FilePath.lean index 4a8c5dc76d1f..18f9d6321327 100644 --- a/src/Init/System/FilePath.lean +++ b/src/Init/System/FilePath.lean @@ -5,8 +5,6 @@ Authors: Leonardo de Moura, Sebastian Ullrich -/ prelude import Init.System.Platform -import Init.Data.String.Basic -import Init.Data.Repr import Init.Data.ToString.Basic namespace System diff --git a/src/Init/System/IO.lean b/src/Init/System/IO.lean index f391dedec4fc..15b0d8c58391 100644 --- a/src/Init/System/IO.lean +++ b/src/Init/System/IO.lean @@ -4,13 +4,9 @@ Released under Apache 2.0 license as described in the file LICENSE. Authors: Luke Nelson, Jared Roesch, Leonardo de Moura, Sebastian Ullrich, Mac Malone -/ prelude -import Init.Control.Reader -import Init.Data.String -import Init.Data.ByteArray import Init.System.IOError import Init.System.FilePath import Init.System.ST -import Init.Data.ToString.Macro import Init.Data.Ord open System diff --git a/src/Init/System/IOError.lean b/src/Init/System/IOError.lean index 4e76bb964ee1..4068503078c1 100644 --- a/src/Init/System/IOError.lean +++ b/src/Init/System/IOError.lean @@ -5,10 +5,7 @@ Authors: Simon Hudon -/ prelude -import Init.Core -import Init.Data.UInt.Basic import Init.Data.ToString.Basic -import Init.Data.String.Basic /-- Imitate the structure of IOErrorType in Haskell: diff --git a/src/Init/Tactics.lean b/src/Init/Tactics.lean index 72e333f66f72..389010b828b2 100644 --- a/src/Init/Tactics.lean +++ b/src/Init/Tactics.lean @@ -495,7 +495,7 @@ macro (name := rwSeq) "rw " c:(config)? s:rwRuleSeq l:(location)? : tactic => `(tactic| (rewrite $(c)? [$rs,*] $(l)?; with_annotate_state $rbrak (try (with_reducible rfl)))) | _ => Macro.throwUnsupported -/-- `rwa` calls `rw`, then closes any remaining goals using `assumption`. -/ +/-- `rwa` is short-hand for `rw; assumption`. -/ macro "rwa " rws:rwRuleSeq loc:(location)? : tactic => `(tactic| (rw $rws:rwRuleSeq $[$loc:location]?; assumption)) diff --git a/src/Lean/Declaration.lean b/src/Lean/Declaration.lean index 4be29c41349c..b764111ddaa9 100644 --- a/src/Lean/Declaration.lean +++ b/src/Lean/Declaration.lean @@ -472,6 +472,10 @@ def isInductive : ConstantInfo → Bool | inductInfo _ => true | _ => false +def isTheorem : ConstantInfo → Bool + | thmInfo _ => true + | _ => false + def inductiveVal! : ConstantInfo → InductiveVal | .inductInfo val => val | _ => panic! "Expected a `ConstantInfo.inductInfo`." diff --git a/src/Lean/Elab/BuiltinCommand.lean b/src/Lean/Elab/BuiltinCommand.lean index 66d21a068ffa..79295519a126 100644 --- a/src/Lean/Elab/BuiltinCommand.lean +++ b/src/Lean/Elab/BuiltinCommand.lean @@ -343,7 +343,7 @@ def failIfSucceeds (x : CommandElabM Unit) : CommandElabM Unit := do if let .none ← findDeclarationRangesCore? declName then -- this is only relevant for declarations added without a declaration range -- in particular `Quot.mk` et al which are added by `init_quot` - addAuxDeclarationRanges declName stx id + addDeclarationRangesFromSyntax declName stx id addDocString declName (← getDocStringText doc) | _ => throwUnsupportedSyntax diff --git a/src/Lean/Elab/BuiltinEvalCommand.lean b/src/Lean/Elab/BuiltinEvalCommand.lean index 659908dda23f..3a11ed0fd81f 100644 --- a/src/Lean/Elab/BuiltinEvalCommand.lean +++ b/src/Lean/Elab/BuiltinEvalCommand.lean @@ -84,7 +84,7 @@ private def addAndCompileExprForEval (declName : Name) (value : Expr) (allowSorr -- An alternative design would be to make `elabTermForEval` into a term elaborator and elaborate the command all at once -- with `unsafe def _eval := term_for_eval% $t`, which we did try, but unwanted error messages -- such as "failed to infer definition type" can surface. - let defView := mkDefViewOfDef { isUnsafe := true, stx := ⟨.missing⟩ } + let defView := mkDefViewOfDef { isUnsafe := true } (← `(Parser.Command.definition| def $(mkIdent <| `_root_ ++ declName) := $(← Term.exprToSyntax value))) Term.elabMutualDef #[] { header := "" } #[defView] diff --git a/src/Lean/Elab/Command.lean b/src/Lean/Elab/Command.lean index e73c8c67514b..296a2bede02f 100644 --- a/src/Lean/Elab/Command.lean +++ b/src/Lean/Elab/Command.lean @@ -711,21 +711,54 @@ def addUnivLevel (idStx : Syntax) : CommandElabM Unit := withRef idStx do else modifyScope fun scope => { scope with levelNames := id :: scope.levelNames } -def expandDeclId (declId : Syntax) (modifiers : Modifiers) : CommandElabM ExpandDeclIdResult := do - let currNamespace ← getCurrNamespace - let currLevelNames ← getLevelNames - let r ← Elab.expandDeclId currNamespace currLevelNames declId modifiers - for id in (← (← getScope).varDecls.flatMapM getBracketedBinderIds) do - if id == r.shortName then - throwError "invalid declaration name '{r.shortName}', there is a section variable with the same name" - return r - end Elab.Command open Elab Command MonadRecDepth +private def liftCommandElabMCore (cmd : CommandElabM α) (throwOnError : Bool) : CoreM α := do + let s : Core.State ← get + let ctx : Core.Context ← read + let (a, commandState) ← + cmd.run { + fileName := ctx.fileName + fileMap := ctx.fileMap + currRecDepth := ctx.currRecDepth + currMacroScope := ctx.currMacroScope + ref := ctx.ref + tacticCache? := none + snap? := none + cancelTk? := ctx.cancelTk? + suppressElabErrors := ctx.suppressElabErrors + } |>.run { + env := s.env + nextMacroScope := s.nextMacroScope + maxRecDepth := ctx.maxRecDepth + ngen := s.ngen + scopes := [{ header := "", opts := ctx.options }] + infoState.enabled := s.infoState.enabled + } + modify fun coreState => { coreState with + env := commandState.env + nextMacroScope := commandState.nextMacroScope + ngen := commandState.ngen + traceState.traces := coreState.traceState.traces ++ commandState.traceState.traces + } + if throwOnError then + if let some err := commandState.messages.toArray.find? (·.severity matches .error) then + throwError err.data + modify fun coreState => { coreState with + infoState.trees := coreState.infoState.trees.append commandState.infoState.trees + messages := coreState.messages ++ commandState.messages + } + return a + /-- -Lifts an action in `CommandElabM` into `CoreM`, updating the traces and the environment. +Lifts an action in `CommandElabM` into `CoreM`, updating the environment, +messages, info trees, traces, the name generator, and macro scopes. +The action is run in a context with an empty message log, empty trace state, and empty info trees. + +If `throwOnError` is true, then if the command produces an error message, it is converted into an exception. +In this case, info trees and messages are not carried over. Commands that modify the processing of subsequent commands, such as `open` and `namespace` commands, @@ -738,27 +771,9 @@ to reset the instance cache. While the `modifyEnv` function for `MetaM` clears its caches entirely, `liftCommandElabM` has no way to reset these caches. -/ -def liftCommandElabM (cmd : CommandElabM α) : CoreM α := do - let (a, commandState) ← - cmd.run { - fileName := ← getFileName - fileMap := ← getFileMap - ref := ← getRef - tacticCache? := none - snap? := none - cancelTk? := (← read).cancelTk? - } |>.run { - env := ← getEnv - maxRecDepth := ← getMaxRecDepth - scopes := [{ header := "", opts := ← getOptions }] - } - modify fun coreState => { coreState with - traceState.traces := coreState.traceState.traces ++ commandState.traceState.traces - env := commandState.env - } - if let some err := commandState.messages.toArray.find? (·.severity matches .error) then - throwError err.data - pure a +def liftCommandElabM (cmd : CommandElabM α) (throwOnError : Bool := true) : CoreM α := do + -- `observing` ensures that if `cmd` throws an exception we still thread state back to `CoreM`. + MonadExcept.ofExcept (← liftCommandElabMCore (observing cmd) throwOnError) /-- Given a command elaborator `cmd`, returns a new command elaborator that diff --git a/src/Lean/Elab/DeclModifiers.lean b/src/Lean/Elab/DeclModifiers.lean index 55db381c1a40..a6c86a04e744 100644 --- a/src/Lean/Elab/DeclModifiers.lean +++ b/src/Lean/Elab/DeclModifiers.lean @@ -57,7 +57,8 @@ inductive RecKind where /-- Flags and data added to declarations (eg docstrings, attributes, `private`, `unsafe`, `partial`, ...). -/ structure Modifiers where - stx : TSyntax ``Parser.Command.declModifiers + /-- Input syntax, used for adjusting declaration range (unless missing) -/ + stx : TSyntax ``Parser.Command.declModifiers := ⟨.missing⟩ docString? : Option String := none visibility : Visibility := Visibility.regular isNoncomputable : Bool := false diff --git a/src/Lean/Elab/Declaration.lean b/src/Lean/Elab/Declaration.lean index 21c01998a88a..33a7dcf9218c 100644 --- a/src/Lean/Elab/Declaration.lean +++ b/src/Lean/Elab/Declaration.lean @@ -102,14 +102,16 @@ def elabAxiom (modifiers : Modifiers) (stx : Syntax) : CommandElabM Unit := do -- leading_parser "axiom " >> declId >> declSig let declId := stx[1] let (binders, typeStx) := expandDeclSig stx[2] - let scopeLevelNames ← getLevelNames - let ⟨_, declName, allUserLevelNames⟩ ← expandDeclId declId modifiers - addDeclarationRanges declName modifiers.stx stx - runTermElabM fun vars => + runTermElabM fun vars => do + let scopeLevelNames ← Term.getLevelNames + let ⟨shortName, declName, allUserLevelNames⟩ ← Term.expandDeclId (← getCurrNamespace) scopeLevelNames declId modifiers + addDeclarationRangesForBuiltin declName modifiers.stx stx + Term.withAutoBoundImplicitForbiddenPred (fun n => shortName == n) do Term.withDeclName declName <| Term.withLevelNames allUserLevelNames <| Term.elabBinders binders.getArgs fun xs => do Term.applyAttributesAt declName modifiers.attrs AttributeApplicationTime.beforeElaboration let type ← Term.elabType typeStx Term.synthesizeSyntheticMVarsNoPostponing + let xs ← Term.addAutoBoundImplicits xs let type ← instantiateMVars type let type ← mkForallFVars xs type let type ← mkForallFVars vars type (usedOnly := true) @@ -135,63 +137,6 @@ def elabAxiom (modifiers : Modifiers) (stx : Syntax) : CommandElabM Unit := do compileDecl decl Term.applyAttributesAt declName modifiers.attrs AttributeApplicationTime.afterCompilation -/- -leading_parser "inductive " >> declId >> optDeclSig >> optional ("where" <|> ":=") >> many ctor -leading_parser atomic (group ("class " >> "inductive ")) >> declId >> optDeclSig >> optional ("where" <|> ":=") >> many ctor >> optDeriving --/ -private def inductiveSyntaxToView (modifiers : Modifiers) (decl : Syntax) : CommandElabM InductiveView := do - checkValidInductiveModifier modifiers - let (binders, type?) := expandOptDeclSig decl[2] - let declId := decl[1] - let ⟨name, declName, levelNames⟩ ← expandDeclId declId modifiers - addDeclarationRanges declName modifiers.stx decl - let ctors ← decl[4].getArgs.mapM fun ctor => withRef ctor do - -- def ctor := leading_parser optional docComment >> "\n| " >> declModifiers >> rawIdent >> optDeclSig - let mut ctorModifiers ← elabModifiers ⟨ctor[2]⟩ - if let some leadingDocComment := ctor[0].getOptional? then - if ctorModifiers.docString?.isSome then - logErrorAt leadingDocComment "duplicate doc string" - ctorModifiers := { ctorModifiers with docString? := TSyntax.getDocString ⟨leadingDocComment⟩ } - if ctorModifiers.isPrivate && modifiers.isPrivate then - throwError "invalid 'private' constructor in a 'private' inductive datatype" - if ctorModifiers.isProtected && modifiers.isPrivate then - throwError "invalid 'protected' constructor in a 'private' inductive datatype" - checkValidCtorModifier ctorModifiers - let ctorName := ctor.getIdAt 3 - let ctorName := declName ++ ctorName - let ctorName ← withRef ctor[3] <| applyVisibility ctorModifiers.visibility ctorName - let (binders, type?) := expandOptDeclSig ctor[4] - addDocString' ctorName ctorModifiers.docString? - addAuxDeclarationRanges ctorName ctor ctor[3] - return { ref := ctor, modifiers := ctorModifiers, declName := ctorName, binders := binders, type? := type? : CtorView } - let 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]⟩ } - let classes ← liftCoreM <| getOptDerivingClasses decl[6] - if decl[3][0].isToken ":=" then - -- https://github.com/leanprover/lean4/issues/5236 - withRef decl[0] <| Linter.logLintIf Linter.linter.deprecated decl[3] - "'inductive ... :=' has been deprecated in favor of 'inductive ... where'." - return { - ref := decl - shortDeclName := name - derivingClasses := classes - declId, modifiers, declName, levelNames - binders, type?, ctors - computedFields - } - -private def classInductiveSyntaxToView (modifiers : Modifiers) (decl : Syntax) : CommandElabM InductiveView := - inductiveSyntaxToView modifiers decl - -def elabInductive (modifiers : Modifiers) (stx : Syntax) : CommandElabM Unit := do - let v ← inductiveSyntaxToView modifiers stx - elabInductiveViews #[v] - -def elabClassInductive (modifiers : Modifiers) (stx : Syntax) : CommandElabM Unit := do - let modifiers := modifiers.addAttr { name := `class } - let v ← classInductiveSyntaxToView modifiers stx - elabInductiveViews #[v] - /-- Macro that expands a declaration with a complex name into an explicit `namespace` block. Implementing this step as a macro means that reuse checking is handled by `elabCommand`. @@ -230,19 +175,6 @@ def elabDeclaration : CommandElab := fun stx => do else throwError "unexpected declaration" -/-- 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] - let declKind := decl.getKind - declKind == `Lean.Parser.Command.inductive - -private def elabMutualInductive (elems : Array Syntax) : CommandElabM Unit := do - let views ← elems.mapM fun stx => do - let modifiers ← elabModifiers ⟨stx[0]⟩ - inductiveSyntaxToView modifiers stx[1] - elabInductiveViews views - /-- 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 => @@ -400,7 +332,7 @@ def elabMutual : CommandElab := fun stx => do -- We need to add `id`'s ranges *before* elaborating `initFn` (and then `id` itself) as -- otherwise the info context created by `with_decl_name` will be incomplete and break the -- call hierarchy - addDeclarationRanges fullId ⟨defStx.raw[0]⟩ defStx.raw[1] + addDeclarationRangesForBuiltin fullId ⟨defStx.raw[0]⟩ defStx.raw[1] elabCommand (← `( $[unsafe%$unsafe?]? def initFn : IO $type := with_decl_name% $(mkIdent fullId) do $doSeq $defStx:command)) diff --git a/src/Lean/Elab/DeclarationRange.lean b/src/Lean/Elab/DeclarationRange.lean index 610fad80a339..44e08e263cbf 100644 --- a/src/Lean/Elab/DeclarationRange.lean +++ b/src/Lean/Elab/DeclarationRange.lean @@ -49,29 +49,31 @@ def getDeclarationSelectionRef (stx : Syntax) : Syntax := else stx[0] +/-- +Derives and adds declaration ranges from given syntax trees. If `rangeStx` does not have a range, +nothing is added. If `selectionRangeStx` does not have a range, it is defaulted to that of +`rangeStx`. +-/ +def addDeclarationRangesFromSyntax [Monad m] [MonadEnv m] [MonadFileMap m] (declName : Name) + (rangeStx : Syntax) (selectionRangeStx : Syntax := .missing) : m Unit := do + -- may fail on partial syntax, ignore in that case + let some range ← getDeclarationRange? rangeStx | return + let selectionRange ← (·.getD range) <$> getDeclarationRange? selectionRangeStx + Lean.addDeclarationRanges declName { range, selectionRange } /-- Stores the `range` and `selectionRange` for `declName` where `modsStx` is the modifier part and `cmdStx` the remaining part of the syntax tree for `declName`. This method is for the builtin declarations only. User-defined commands should use -`Lean.addDeclarationRanges` to store this information for their commands. +`Lean.Elab.addDeclarationRangesFromSyntax` or `Lean.addDeclarationRanges` to store this information +for their commands. -/ -def addDeclarationRanges [Monad m] [MonadEnv m] [MonadFileMap m] (declName : Name) +def addDeclarationRangesForBuiltin [Monad m] [MonadEnv m] [MonadFileMap m] (declName : Name) (modsStx : TSyntax ``Parser.Command.declModifiers) (declStx : Syntax) : m Unit := do if declStx.getKind == ``Parser.Command.«example» then return () let stx := mkNullNode #[modsStx, declStx] - -- may fail on partial syntax, ignore in that case - let some range ← getDeclarationRange? stx | return - let some selectionRange ← getDeclarationRange? (getDeclarationSelectionRef declStx) | return - Lean.addDeclarationRanges declName { range, selectionRange } - -/-- Auxiliary method for recording ranges for auxiliary declarations (e.g., fields, nested declarations, etc. -/ -def addAuxDeclarationRanges [Monad m] [MonadEnv m] [MonadFileMap m] (declName : Name) (stx : Syntax) (header : Syntax) : m Unit := do - -- may fail on partial syntax, ignore in that case - let some range ← getDeclarationRange? stx | return - let some selectionRange ← getDeclarationRange? header | return - Lean.addDeclarationRanges declName { range, selectionRange } + addDeclarationRangesFromSyntax declName stx (getDeclarationSelectionRef declStx) end Lean.Elab diff --git a/src/Lean/Elab/Frontend.lean b/src/Lean/Elab/Frontend.lean index 0a248a42a7d4..132a7a32c3fb 100644 --- a/src/Lean/Elab/Frontend.lean +++ b/src/Lean/Elab/Frontend.lean @@ -145,7 +145,7 @@ def runFrontend : IO (Environment × Bool) := do let startTime := (← IO.monoNanosNow).toFloat / 1000000000 let inputCtx := Parser.mkInputContext input fileName - let opts := Language.Lean.internal.cmdlineSnapshots.set opts true + let opts := Language.Lean.internal.cmdlineSnapshots.setIfNotSet opts true let ctx := { inputCtx with } let processor := Language.Lean.process let snap ← processor (fun _ => pure <| .ok { mainModuleName, opts, trustLevel }) none ctx diff --git a/src/Lean/Elab/Inductive.lean b/src/Lean/Elab/Inductive.lean index 0ddb49ce0cf3..cb59576744d6 100644 --- a/src/Lean/Elab/Inductive.lean +++ b/src/Lean/Elab/Inductive.lean @@ -18,6 +18,7 @@ import Lean.Elab.ComputedFields import Lean.Elab.DefView import Lean.Elab.DeclUtil import Lean.Elab.Deriving.Basic +import Lean.Elab.DeclarationRange namespace Lean.Elab.Command open Meta @@ -79,10 +80,56 @@ structure ElabHeaderResult where view : InductiveView lctx : LocalContext localInsts : LocalInstances + levelNames : List Name params : Array Expr type : Expr deriving Inhabited +/- +leading_parser "inductive " >> declId >> optDeclSig >> optional ("where" <|> ":=") >> many ctor +leading_parser atomic (group ("class " >> "inductive ")) >> declId >> optDeclSig >> optional ("where" <|> ":=") >> many ctor >> optDeriving +-/ +private def inductiveSyntaxToView (modifiers : Modifiers) (decl : Syntax) : TermElabM InductiveView := do + checkValidInductiveModifier modifiers + let (binders, type?) := expandOptDeclSig decl[2] + let declId := decl[1] + let ⟨name, declName, levelNames⟩ ← Term.expandDeclId (← getCurrNamespace) (← Term.getLevelNames) declId modifiers + addDeclarationRangesForBuiltin declName modifiers.stx decl + let ctors ← decl[4].getArgs.mapM fun ctor => withRef ctor do + -- def ctor := leading_parser optional docComment >> "\n| " >> declModifiers >> rawIdent >> optDeclSig + let mut ctorModifiers ← elabModifiers ⟨ctor[2]⟩ + if let some leadingDocComment := ctor[0].getOptional? then + if ctorModifiers.docString?.isSome then + logErrorAt leadingDocComment "duplicate doc string" + ctorModifiers := { ctorModifiers with docString? := TSyntax.getDocString ⟨leadingDocComment⟩ } + if ctorModifiers.isPrivate && modifiers.isPrivate then + throwError "invalid 'private' constructor in a 'private' inductive datatype" + if ctorModifiers.isProtected && modifiers.isPrivate then + throwError "invalid 'protected' constructor in a 'private' inductive datatype" + checkValidCtorModifier ctorModifiers + let ctorName := ctor.getIdAt 3 + let ctorName := declName ++ ctorName + let ctorName ← withRef ctor[3] <| applyVisibility ctorModifiers.visibility ctorName + let (binders, type?) := expandOptDeclSig ctor[4] + addDocString' ctorName ctorModifiers.docString? + addDeclarationRangesFromSyntax ctorName ctor ctor[3] + return { ref := ctor, modifiers := ctorModifiers, declName := ctorName, binders := binders, type? := type? : CtorView } + let 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]⟩ } + let classes ← getOptDerivingClasses decl[6] + if decl[3][0].isToken ":=" then + -- https://github.com/leanprover/lean4/issues/5236 + withRef decl[0] <| Linter.logLintIf Linter.linter.deprecated decl[3] + "'inductive ... :=' has been deprecated in favor of 'inductive ... where'." + return { + ref := decl + shortDeclName := name + derivingClasses := classes + declId, modifiers, declName, levelNames + binders, type?, ctors + computedFields + } + private partial def elabHeaderAux (views : Array InductiveView) (i : Nat) (acc : Array ElabHeaderResult) : TermElabM (Array ElabHeaderResult) := Term.withAutoBoundImplicitForbiddenPred (fun n => views.any (·.shortDeclName == n)) do if h : i < views.size then @@ -94,7 +141,8 @@ private partial def elabHeaderAux (views : Array InductiveView) (i : Nat) (acc : let type := mkSort u Term.synthesizeSyntheticMVarsNoPostponing Term.addAutoBoundImplicits' params type fun params type => do - return acc.push { lctx := (← getLCtx), localInsts := (← getLocalInstances), params, type, view } + let levelNames ← Term.getLevelNames + return acc.push { lctx := (← getLCtx), localInsts := (← getLocalInstances), levelNames, params, type, view } | some typeStx => let (type, _) ← Term.withAutoBoundImplicit do let type ← Term.elabType typeStx @@ -105,7 +153,8 @@ private partial def elabHeaderAux (views : Array InductiveView) (i : Nat) (acc : return (← mkForallFVars indices type, indices.size) Term.addAutoBoundImplicits' params type fun params type => do trace[Elab.inductive] "header params: {params}, type: {type}" - return acc.push { lctx := (← getLCtx), localInsts := (← getLocalInstances), params, type, view } + let levelNames ← Term.getLevelNames + return acc.push { lctx := (← getLCtx), localInsts := (← getLocalInstances), levelNames, params, type, view } elabHeaderAux views (i+1) acc else return acc @@ -123,13 +172,20 @@ private def checkUnsafe (rs : Array ElabHeaderResult) : TermElabM Unit := do unless r.view.modifiers.isUnsafe == isUnsafe do throwErrorAt r.view.ref "invalid inductive type, cannot mix unsafe and safe declarations in a mutually inductive datatypes" -private def checkLevelNames (views : Array InductiveView) : TermElabM Unit := do +private def InductiveView.checkLevelNames (views : Array InductiveView) : TermElabM Unit := do if views.size > 1 then let levelNames := views[0]!.levelNames for view in views do unless view.levelNames == levelNames do throwErrorAt view.ref "invalid inductive type, universe parameters mismatch in mutually inductive datatypes" +private def ElabHeaderResult.checkLevelNames (rs : Array ElabHeaderResult) : TermElabM Unit := do + if rs.size > 1 then + let levelNames := rs[0]!.levelNames + for r in rs do + unless r.levelNames == levelNames do + throwErrorAt r.view.ref "invalid inductive type, universe parameters mismatch in mutually inductive datatypes" + private def mkTypeFor (r : ElabHeaderResult) : TermElabM Expr := do withLCtx r.lctx r.localInsts do mkForallFVars r.params r.type @@ -791,12 +847,15 @@ private partial def fixedIndicesToParams (numParams : Nat) (indTypes : Array Ind private def mkInductiveDecl (vars : Array Expr) (views : Array InductiveView) : TermElabM Unit := Term.withoutSavingRecAppSyntax do let view0 := views[0]! let scopeLevelNames ← Term.getLevelNames - checkLevelNames views + InductiveView.checkLevelNames views let allUserLevelNames := view0.levelNames let isUnsafe := view0.modifiers.isUnsafe withRef view0.ref <| Term.withLevelNames allUserLevelNames do let rs ← elabHeader views Term.synthesizeSyntheticMVarsNoPostponing + ElabHeaderResult.checkLevelNames rs + let allUserLevelNames := rs[0]!.levelNames + trace[Elab.inductive] "level names: {allUserLevelNames}" withInductiveLocalDecls rs fun params indFVars => do trace[Elab.inductive] "indFVars: {indFVars}" let mut indTypesArray := #[] @@ -888,19 +947,55 @@ private def applyComputedFields (indViews : Array InductiveView) : CommandElabM liftTermElabM do Term.withDeclName indViews[0]!.declName do ComputedFields.setComputedFields computedFields -def elabInductiveViews (views : Array InductiveView) : CommandElabM Unit := do +def elabInductiveViews (vars : Array Expr) (views : Array InductiveView) : TermElabM Unit := do let view0 := views[0]! let ref := view0.ref - runTermElabM fun vars => Term.withDeclName view0.declName do withRef ref do + Term.withDeclName view0.declName do withRef ref do mkInductiveDecl vars views mkSizeOfInstances view0.declName Lean.Meta.IndPredBelow.mkBelow view0.declName for view in views do mkInjectiveTheorems view.declName + +def elabInductiveViewsPostprocessing (views : Array InductiveView) : CommandElabM Unit := do + let view0 := views[0]! + let ref := view0.ref applyComputedFields views -- NOTE: any generated code before this line is invalid applyDerivingHandlers views runTermElabM fun _ => Term.withDeclName view0.declName do withRef ref do for view in views do Term.applyAttributesAt view.declName view.modifiers.attrs .afterCompilation +def elabInductives (inductives : Array (Modifiers × Syntax)) : CommandElabM Unit := do + let vs ← runTermElabM fun vars => do + let vs ← inductives.mapM fun (modifiers, stx) => inductiveSyntaxToView modifiers stx + elabInductiveViews vars vs + pure vs + elabInductiveViewsPostprocessing vs + +def elabInductive (modifiers : Modifiers) (stx : Syntax) : CommandElabM Unit := do + elabInductives #[(modifiers, stx)] + +def elabClassInductive (modifiers : Modifiers) (stx : Syntax) : CommandElabM Unit := do + let modifiers := modifiers.addAttr { name := `class } + elabInductive modifiers stx + +/-- +Returns true if all elements of the `mutual` block (`Lean.Parser.Command.mutual`) are inductive declarations. +-/ +def isMutualInductive (stx : Syntax) : Bool := + stx[1].getArgs.all fun elem => + let decl := elem[1] + let declKind := decl.getKind + declKind == `Lean.Parser.Command.inductive + +/-- +Elaborates a `mutual` block satisfying `Lean.Elab.Command.isMutualInductive`. +-/ +def elabMutualInductive (elems : Array Syntax) : CommandElabM Unit := do + let inductives ← elems.mapM fun stx => do + let modifiers ← elabModifiers ⟨stx[0]⟩ + pure (modifiers, stx[1]) + elabInductives inductives + end Lean.Elab.Command diff --git a/src/Lean/Elab/LetRec.lean b/src/Lean/Elab/LetRec.lean index 64b8b9f61141..32c3d4abc0a7 100644 --- a/src/Lean/Elab/LetRec.lean +++ b/src/Lean/Elab/LetRec.lean @@ -51,7 +51,7 @@ private def mkLetRecDeclView (letRec : Syntax) : TermElabM LetRecView := do checkNotAlreadyDeclared declName applyAttributesAt declName attrs AttributeApplicationTime.beforeElaboration addDocString' declName docStr? - addAuxDeclarationRanges declName decl declId + addDeclarationRangesFromSyntax declName decl declId let binders := decl[1].getArgs let typeStx := expandOptType declId decl[2] let (type, binderIds) ← elabBindersEx binders fun xs => do diff --git a/src/Lean/Elab/MutualDef.lean b/src/Lean/Elab/MutualDef.lean index a4646595d55b..ccb1af447708 100644 --- a/src/Lean/Elab/MutualDef.lean +++ b/src/Lean/Elab/MutualDef.lean @@ -887,7 +887,6 @@ def getKindForLetRecs (mainHeaders : Array DefViewElabHeader) : DefKind := else DefKind.«def» def getModifiersForLetRecs (mainHeaders : Array DefViewElabHeader) : Modifiers := { - stx := ⟨mkNullNode #[]⟩ -- ignore when computing declaration range isNoncomputable := mainHeaders.any fun h => h.modifiers.isNoncomputable recKind := if mainHeaders.any fun h => h.modifiers.isPartial then RecKind.partial else RecKind.default isUnsafe := mainHeaders.any fun h => h.modifiers.isUnsafe @@ -998,7 +997,7 @@ where for view in views, header in headers do -- NOTE: this should be the full `ref`, and thus needs to be done after any snapshotting -- that depends only on a part of the ref - addDeclarationRanges header.declName view.modifiers.stx view.ref + addDeclarationRangesForBuiltin header.declName view.modifiers.stx view.ref processDeriving (headers : Array DefViewElabHeader) := do diff --git a/src/Lean/Elab/PreDefinition/MkInhabitant.lean b/src/Lean/Elab/PreDefinition/MkInhabitant.lean index ec50b443d8d7..910a2268a17a 100644 --- a/src/Lean/Elab/PreDefinition/MkInhabitant.lean +++ b/src/Lean/Elab/PreDefinition/MkInhabitant.lean @@ -5,9 +5,24 @@ Authors: Leonardo de Moura -/ prelude import Lean.Meta.AppBuilder +import Lean.PrettyPrinter namespace Lean.Elab open Meta +private def withInhabitedInstances (xs : Array Expr) (k : Array Expr → MetaM α) : MetaM α := do + let rec go (i : Nat) (insts : Array Expr) : MetaM α := do + if h : i < xs.size then + let x := xs[i] + let xTy ← inferType x + let u ← getLevel xTy + let instTy := mkApp (.const ``Inhabited [u]) xTy + let instVal := mkApp2 (.const ``Inhabited.mk [u]) xTy x + withLetDecl `inst instTy instVal fun inst => + go (i + 1) (insts.push inst) + else + k insts + go 0 #[] + private def mkInhabitant? (type : Expr) (useOfNonempty : Bool) : MetaM (Option Expr) := do try if useOfNonempty then @@ -17,36 +32,41 @@ private def mkInhabitant? (type : Expr) (useOfNonempty : Bool) : MetaM (Option E catch _ => return none -private def findAssumption? (xs : Array Expr) (type : Expr) : MetaM (Option Expr) := do - xs.findM? fun x => do isDefEq (← inferType x) type - -private def mkFnInhabitant? (xs : Array Expr) (type : Expr) (useOfNonempty : Bool) : MetaM (Option Expr) := - let rec loop - | 0, type => mkInhabitant? type useOfNonempty - | i+1, type => do - let x := xs[i]! - let type ← mkForallFVars #[x] type; - match (← mkInhabitant? type useOfNonempty) with - | none => loop i type - | some val => return some (← mkLambdaFVars xs[0:i] val) - loop xs.size type +/-- +Find an inhabitant while doing delta unfolding. +-/ +private partial def mkInhabitantForAux? (xs insts : Array Expr) (type : Expr) (useOfNonempty : Bool) : MetaM (Option Expr) := withIncRecDepth do + if let some val ← mkInhabitant? type useOfNonempty then + mkLambdaFVars xs (← mkLetFVars (usedLetOnly := true) insts val) + else + let type ← whnfCore type + if type.isForall then + forallTelescope type fun xs' type' => + withInhabitedInstances xs' fun insts' => + mkInhabitantForAux? (xs ++ xs') (insts ++ insts') type' useOfNonempty + else if let some type' ← unfoldDefinition? type then + mkInhabitantForAux? xs insts type' useOfNonempty + else + return none /- 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 - | some val => mkLambdaFVars xs val - | none => - match (← findAssumption? xs type) with - | some x => mkLambdaFVars xs x - | none => - match (← mkFnInhabitant? xs type useOfNonempty) with - | some val => return val - | none => return none - match (← go? false) with - | some val => return val - | none => match (← go? true) with - | some val => return val - | none => throwError "failed to compile partial definition '{declName}', failed to show that type is inhabited and non empty" +def mkInhabitantFor (declName : Name) (xs : Array Expr) (type : Expr) : MetaM Expr := + withInhabitedInstances xs fun insts => do + if let some val ← mkInhabitantForAux? xs insts type false <||> mkInhabitantForAux? xs insts type true then + return val + else + throwError "\ + failed to compile 'partial' definition '{declName}', could not prove that the type\ + {indentExpr (← mkForallFVars xs type)}\n\ + is nonempty.\n\ + \n\ + This process uses multiple strategies:\n\ + - It looks for a parameter that matches the return type.\n\ + - It tries synthesizing '{MessageData.ofConstName ``Inhabited}' and '{MessageData.ofConstName ``Nonempty}' \ + instances for the return type, while making every parameter into a local '{MessageData.ofConstName ``Inhabited}' instance.\n\ + - It tries unfolding the return type.\n\ + \n\ + If the return type is defined using the 'structure' or 'inductive' command, \ + you can try adding a 'deriving Nonempty' clause to it." end Lean.Elab diff --git a/src/Lean/Elab/StructInst.lean b/src/Lean/Elab/StructInst.lean index ca64cd377749..dba423d24207 100644 --- a/src/Lean/Elab/StructInst.lean +++ b/src/Lean/Elab/StructInst.lean @@ -826,9 +826,12 @@ def mkDefaultValue? (struct : Struct) (cinfo : ConstantInfo) : TermElabM (Option /-- Reduce default value. It performs beta reduction and projections of the given structures. -/ partial def reduce (structNames : Array Name) (e : Expr) : MetaM Expr := do match e with - | .lam .. => lambdaLetTelescope e fun xs b => do mkLambdaFVars xs (← reduce structNames b) - | .forallE .. => forallTelescope e fun xs b => do mkForallFVars xs (← reduce structNames b) - | .letE .. => lambdaLetTelescope e fun xs b => do mkLetFVars xs (← reduce structNames b) + | .forallE .. => + forallTelescope e fun xs b => withReduceLCtx xs do + mkForallFVars xs (← reduce structNames b) + | .lam .. | .letE .. => + lambdaLetTelescope e fun xs b => withReduceLCtx xs do + mkLambdaFVars (usedLetOnly := true) xs (← reduce structNames b) | .proj _ i b => match (← Meta.project? b i) with | some r => reduce structNames r @@ -858,6 +861,24 @@ partial def reduce (structNames : Array Name) (e : Expr) : MetaM Expr := do | some val => if val.isMVar then pure val else reduce structNames val | none => return e | e => return e +where + /-- + Reduce the types and values of the local variables `xs` in the local context. + -/ + withReduceLCtx {α} (xs : Array Expr) (k : MetaM α) (i : Nat := 0) : MetaM α := do + if h : i < xs.size then + let fvarId := xs[i].fvarId! + let decl ← fvarId.getDecl + let type ← reduce structNames decl.type + let mut lctx ← getLCtx + if let some value := decl.value? then + let value ← reduce structNames value + lctx := lctx.modifyLocalDecl fvarId (· |>.setType type |>.setValue value) + else + lctx := lctx.modifyLocalDecl fvarId (· |>.setType type) + withLCtx lctx (← getLocalInstances) (withReduceLCtx xs k (i + 1)) + else + k partial def tryToSynthesizeDefault (structs : Array Struct) (allStructNames : Array Name) (maxDistance : Nat) (fieldName : Name) (mvarId : MVarId) : TermElabM Bool := let rec loop (i : Nat) (dist : Nat) := do @@ -873,6 +894,7 @@ partial def tryToSynthesizeDefault (structs : Array Struct) (allStructNames : Ar | none => setMCtx mctx; loop (i+1) (dist+1) | some val => let val ← reduce allStructNames val + trace[Elab.struct] "default value for {fieldName}:{indentExpr val}" match val.find? fun e => (defaultMissing? e).isSome with | some _ => setMCtx mctx; loop (i+1) (dist+1) | none => diff --git a/src/Lean/Elab/Structure.lean b/src/Lean/Elab/Structure.lean index 5f2d4c9034ca..35faf6ef6489 100644 --- a/src/Lean/Elab/Structure.lean +++ b/src/Lean/Elab/Structure.lean @@ -20,6 +20,11 @@ import Lean.Elab.Binders namespace Lean.Elab.Command +register_builtin_option structureDiamondWarning : Bool := { + defValue := false + descr := "enable/disable warning messages for structure diamonds" +} + open Meta open TSyntax.Compat @@ -34,12 +39,15 @@ structure StructCtorView where modifiers : Modifiers name : Name declName : Name + deriving Inhabited structure StructFieldView where ref : Syntax modifiers : Modifiers binderInfo : BinderInfo declName : Name + /-- ref for the field name -/ + nameId : Syntax name : Name -- The field name as it is going to be registered in the kernel. It does not include macroscopes. rawName : Name -- Same as `name` but including macroscopes. binders : Syntax @@ -47,24 +55,35 @@ structure StructFieldView where value? : Option Syntax structure StructView where - ref : Syntax - modifiers : Modifiers - scopeLevelNames : List Name -- All `universe` declarations in the current scope - allUserLevelNames : List Name -- `scopeLevelNames` ++ explicit universe parameters provided in the `structure` command - isClass : Bool - declName : Name - scopeVars : Array Expr -- All `variable` declaration in the current scope - params : Array Expr -- Explicit parameters provided in the `structure` command - parents : Array Syntax - type : Syntax - ctor : StructCtorView - fields : Array StructFieldView + ref : Syntax + declId : Syntax + modifiers : Modifiers + isClass : Bool -- struct-only + shortDeclName : Name + declName : Name + levelNames : List Name + binders : Syntax + type : Syntax -- modified (inductive has type?) + parents : Array Syntax -- struct-only + ctor : StructCtorView -- struct-only + fields : Array StructFieldView -- struct-only + derivingClasses : Array DerivingClassView + deriving Inhabited + +structure StructParentInfo where + ref : Syntax + fvar? : Option Expr + structName : Name + subobject : Bool + type : Expr + deriving Inhabited inductive StructFieldKind where | newField | copiedField | fromParent | subobject deriving Inhabited, DecidableEq, Repr structure StructFieldInfo where + ref : Syntax name : Name declName : Name -- Remark: for `fromParent` fields, `declName` is only relevant in the generation of auxiliary "default value" functions. fvar : Expr @@ -72,6 +91,17 @@ structure StructFieldInfo where value? : Option Expr := none deriving Inhabited, Repr +structure ElabStructHeaderResult where + view : StructView + lctx : LocalContext + localInsts : LocalInstances + levelNames : List Name + params : Array Expr + type : Expr + parents : Array StructParentInfo + parentFieldInfos : Array StructFieldInfo + deriving Inhabited + def StructFieldInfo.isFromParent (info : StructFieldInfo) : Bool := match info.kind with | StructFieldKind.fromParent => true @@ -94,7 +124,7 @@ private def expandCtor (structStx : Syntax) (structModifiers : Modifiers) (struc let useDefault := do let declName := structDeclName ++ defaultCtorName let ref := structStx[1].mkSynthetic - addAuxDeclarationRanges declName ref ref + addDeclarationRangesFromSyntax declName ref pure { ref, modifiers := default, name := defaultCtorName, declName } if structStx[5].isNone then useDefault @@ -115,7 +145,7 @@ private def expandCtor (structStx : Syntax) (structModifiers : Modifiers) (struc let declName := structDeclName ++ name let declName ← applyVisibility ctorModifiers.visibility declName addDocString' declName ctorModifiers.docString? - addAuxDeclarationRanges declName ctor[1] ctor[1] + addDeclarationRangesFromSyntax declName ctor[1] pure { ref := ctor[1], name, modifiers := ctorModifiers, declName } def checkValidFieldModifier (modifiers : Modifiers) : TermElabM Unit := do @@ -161,14 +191,15 @@ private def expandFields (structStx : Syntax) (structModifiers : Modifiers) (str throwError "invalid 'private' field in a 'private' structure" if fieldModifiers.isProtected && structModifiers.isPrivate then throwError "invalid 'protected' field in a 'private' structure" - let (binders, type?) ← + let (binders, type?, value?) ← if binfo == BinderInfo.default then let (binders, type?) := expandOptDeclSig fieldBinder[3] let optBinderTacticDefault := fieldBinder[4] if optBinderTacticDefault.isNone then - pure (binders, type?) + pure (binders, type?, none) else if optBinderTacticDefault[0].getKind != ``Parser.Term.binderTactic then - pure (binders, type?) + -- binderDefault := leading_parser " := " >> termParser + pure (binders, type?, some optBinderTacticDefault[0][1]) else let binderTactic := optBinderTacticDefault[0] match type? with @@ -180,22 +211,10 @@ private def expandFields (structStx : Syntax) (structModifiers : Modifiers) (str -- It is safe to reset the binders to a "null" node since there is no value to be elaborated let type ← `(forall $(binders.getArgs):bracketedBinder*, $type) let type ← `(autoParam $type $(mkIdentFrom tac name)) - pure (mkNullNode, some type.raw) + pure (mkNullNode, some type.raw, none) else let (binders, type) := expandDeclSig fieldBinder[3] - pure (binders, some type) - let value? ← if binfo != BinderInfo.default then - pure none - else - let optBinderTacticDefault := fieldBinder[4] - -- trace[Elab.struct] ">>> {optBinderTacticDefault}" - if optBinderTacticDefault.isNone then - pure none - else if optBinderTacticDefault[0].getKind == ``Parser.Term.binderTactic then - pure none - else - -- binderDefault := leading_parser " := " >> termParser - pure (some optBinderTacticDefault[0][1]) + pure (binders, some type, none) let idents := fieldBinder[2].getArgs idents.foldlM (init := views) fun (views : Array StructFieldView) ident => withRef ident do let rawName := ident.getId @@ -211,16 +230,59 @@ private def expandFields (structStx : Syntax) (structModifiers : Modifiers) (str binderInfo := binfo declName name + nameId := ident rawName binders type? value? } -private def validStructType (type : Expr) : Bool := - match type with - | Expr.sort .. => true - | _ => false +/- +leading_parser (structureTk <|> classTk) >> declId >> many Term.bracketedBinder >> optional «extends» >> Term.optType >> + optional (("where" <|> ":=") >> optional structCtor >> structFields) >> optDeriving + +where +def «extends» := leading_parser " extends " >> sepBy1 termParser ", " +def typeSpec := leading_parser " : " >> termParser +def optType : Parser := optional typeSpec + +def structFields := leading_parser many (structExplicitBinder <|> structImplicitBinder <|> structInstBinder) +def structCtor := leading_parser try (declModifiers >> ident >> " :: ") +-/ +def structureSyntaxToView (modifiers : Modifiers) (stx : Syntax) : TermElabM StructView := do + checkValidInductiveModifier modifiers + let isClass := stx[0].getKind == ``Parser.Command.classTk + let modifiers := if isClass then modifiers.addAttr { name := `class } else modifiers + let declId := stx[1] + let ⟨name, declName, levelNames⟩ ← Term.expandDeclId (← getCurrNamespace) (← Term.getLevelNames) declId modifiers + addDeclarationRangesForBuiltin declName modifiers.stx stx + let binders := stx[2] + let exts := stx[3] + let parents := if exts.isNone then #[] else exts[0][1].getSepArgs + let optType := stx[4] + let derivingClasses ← getOptDerivingClasses stx[6] + let type ← if optType.isNone then `(Sort _) else pure optType[0][1] + let ctor ← expandCtor stx modifiers declName + let fields ← expandFields stx modifiers declName + fields.forM fun field => do + if field.declName == ctor.declName then + throwErrorAt field.ref "invalid field name '{field.name}', it is equal to structure constructor name" + addDeclarationRangesFromSyntax field.declName field.ref + return { + ref := stx + declId + modifiers + isClass + shortDeclName := name + declName + levelNames + binders + type + parents + ctor + fields + derivingClasses + } private def findFieldInfo? (infos : Array StructFieldInfo) (fieldName : Name) : Option StructFieldInfo := infos.find? fun info => info.name == fieldName @@ -228,17 +290,12 @@ private def findFieldInfo? (infos : Array StructFieldInfo) (fieldName : Name) : private def containsFieldName (infos : Array StructFieldInfo) (fieldName : Name) : Bool := (findFieldInfo? infos fieldName).isSome -private def updateFieldInfoVal (infos : Array StructFieldInfo) (fieldName : Name) (value : Expr) : Array StructFieldInfo := - infos.map fun info => - if info.name == fieldName then - { info with value? := value } - else +private def replaceFieldInfo (infos : Array StructFieldInfo) (info : StructFieldInfo) : Array StructFieldInfo := + infos.map fun info' => + if info'.name == info.name then info - -register_builtin_option structureDiamondWarning : Bool := { - defValue := false - descr := "enable/disable warning messages for structure diamonds" -} + else + info' /-- Return `some fieldName` if field `fieldName` of the parent structure `parentStructName` is already in `infos` -/ private def findExistingField? (infos : Array StructFieldInfo) (parentStructName : Name) : CoreM (Option Name) := do @@ -259,11 +316,11 @@ where throwError "field '{subfieldName}' from '{parentStructName}' has already been declared" let val ← mkProjection parentFVar subfieldName let type ← inferType val - withLetDecl subfieldName type val fun subfieldFVar => + withLetDecl subfieldName type val fun subfieldFVar => do /- The following `declName` is only used for creating the `_default` auxiliary declaration name when its default value is overwritten in the structure. If the default value is not overwritten, then its value is irrelevant. -/ let declName := structDeclName ++ subfieldName - let infos := infos.push { name := subfieldName, declName, fvar := subfieldFVar, kind := StructFieldKind.fromParent } + let infos := infos.push { ref := (← getRef), name := subfieldName, declName, fvar := subfieldFVar, kind := StructFieldKind.fromParent } go (i+1) infos else k infos @@ -414,7 +471,8 @@ where let fieldDeclName := structDeclName ++ fieldName let fieldDeclName ← applyVisibility (← toVisibility fieldInfo) fieldDeclName addDocString' fieldDeclName (← findDocString? (← getEnv) fieldInfo.projFn) - let infos := infos.push { name := fieldName, declName := fieldDeclName, fvar := fieldFVar, value?, + let infos := infos.push { ref := (← getRef) + name := fieldName, declName := fieldDeclName, fvar := fieldFVar, value?, kind := StructFieldKind.copiedField } copy (i+1) infos fieldMap expandedStructNames if fieldInfo.subobject?.isSome then @@ -428,8 +486,10 @@ where else let subfieldNames := getStructureFieldsFlattened (← getEnv) fieldParentStructName let fieldName := fieldInfo.fieldName - withLocalDecl fieldName fieldInfo.binderInfo fieldType fun parentFVar => - let infos := infos.push { name := fieldName, declName := structDeclName ++ fieldName, fvar := parentFVar, kind := StructFieldKind.subobject } + withLocalDecl fieldName fieldInfo.binderInfo fieldType fun parentFVar => do + let infos := infos.push { ref := (← getRef) + name := fieldName, declName := structDeclName ++ fieldName, fvar := parentFVar, + kind := StructFieldKind.subobject } processSubfields structDeclName parentFVar fieldParentStructName subfieldNames infos fun infos => copy (i+1) infos (fieldMap.insert fieldName parentFVar) expandedStructNames else @@ -466,20 +526,22 @@ private partial def mkToParentName (parentStructName : Name) (p : Name → Bool) if p curr then curr else go (i+1) go 1 -private partial def withParents (view : StructView) (k : Array StructFieldInfo → Array Expr → TermElabM α) : TermElabM α := do +private partial def elabParents (view : StructView) + (k : Array StructFieldInfo → Array StructParentInfo → TermElabM α) : TermElabM α := do go 0 #[] #[] where - go (i : Nat) (infos : Array StructFieldInfo) (copiedParents : Array Expr) : TermElabM α := do + go (i : Nat) (infos : Array StructFieldInfo) (parents : Array StructParentInfo) : TermElabM α := do if h : i < view.parents.size then - let parentStx := view.parents.get ⟨i, h⟩ - withRef parentStx do - let parentType ← Term.withSynthesize <| Term.elabType parentStx - let parentType ← whnf parentType + let parent := view.parents[i] + withRef parent do + let type ← Term.elabType parent + let parentType ← whnf type let parentStructName ← getStructureName parentType if let some existingFieldName ← findExistingField? infos parentStructName then if structureDiamondWarning.get (← getOptions) then logWarning s!"field '{existingFieldName}' from '{parentStructName}' has already been declared" - copyNewFieldsFrom view.declName infos parentType fun infos => go (i+1) infos (copiedParents.push parentType) + let parents := parents.push { ref := parent, fvar? := none, subobject := false, structName := parentStructName, type := parentType } + copyNewFieldsFrom view.declName infos parentType fun infos => go (i+1) infos parents -- TODO: if `class`, then we need to create a let-decl that stores the local instance for the `parentStructure` else let env ← getEnv @@ -487,10 +549,13 @@ where let toParentName := mkToParentName parentStructName fun n => !containsFieldName infos n && !subfieldNames.contains n let binfo := if view.isClass && isClass env parentStructName then BinderInfo.instImplicit else BinderInfo.default withLocalDecl toParentName binfo parentType fun parentFVar => - let infos := infos.push { name := toParentName, declName := view.declName ++ toParentName, fvar := parentFVar, kind := StructFieldKind.subobject } - processSubfields view.declName parentFVar parentStructName subfieldNames infos fun infos => go (i+1) infos copiedParents + let infos := infos.push { ref := parent, + name := toParentName, declName := view.declName ++ toParentName, fvar := parentFVar, + kind := StructFieldKind.subobject } + let parents := parents.push { ref := parent, fvar? := parentFVar, subobject := true, structName := parentStructName, type := parentType } + processSubfields view.declName parentFVar parentStructName subfieldNames infos fun infos => go (i+1) infos parents else - k infos copiedParents + k infos parents private def elabFieldTypeValue (view : StructFieldView) : TermElabM (Option Expr × Option Expr) := Term.withAutoBoundImplicit <| Term.withAutoBoundImplicitForbiddenPred (fun n => view.name == n) <| Term.elabBinders view.binders.getArgs fun params => do @@ -525,7 +590,7 @@ private partial def withFields (views : Array StructFieldView) (infos : Array St where go (i : Nat) (defaultValsOverridden : NameSet) (infos : Array StructFieldInfo) : TermElabM α := do if h : i < views.size then - let view := views.get ⟨i, h⟩ + let view := views[i] withRef view.ref do match findFieldInfo? infos view.name with | none => @@ -534,13 +599,15 @@ where | none, none => throwError "invalid field, type expected" | some type, _ => withLocalDecl view.rawName view.binderInfo type fun fieldFVar => - let infos := infos.push { name := view.name, declName := view.declName, fvar := fieldFVar, value? := value?, + let infos := infos.push { ref := view.nameId + name := view.name, declName := view.declName, fvar := fieldFVar, value? := value?, kind := StructFieldKind.newField } go (i+1) defaultValsOverridden infos | none, some value => let type ← inferType value withLocalDecl view.rawName view.binderInfo type fun fieldFVar => - let infos := infos.push { name := view.name, declName := view.declName, fvar := fieldFVar, value? := value, + let infos := infos.push { ref := view.nameId + name := view.name, declName := view.declName, fvar := fieldFVar, value? := value, kind := StructFieldKind.newField } go (i+1) defaultValsOverridden infos | some info => @@ -560,7 +627,7 @@ where let fvarType ← inferType info.fvar let value ← Term.elabTermEnsuringType valStx fvarType pushInfoLeaf <| .ofFieldRedeclInfo { stx := view.ref } - let infos := updateFieldInfoVal infos info.name value + let infos := replaceFieldInfo infos { info with ref := view.nameId, value? := value } go (i+1) defaultValsOverridden infos match info.kind with | StructFieldKind.newField => throwError "field '{view.name}' has already been declared" @@ -654,13 +721,13 @@ private def updateResultingUniverse (fieldInfos : Array StructFieldInfo) (type : let r ← getResultUniverse type let rOffset : Nat := r.getOffset let r : Level := r.getLevelOffset - match r with - | Level.mvar mvarId => - let us ← collectUniversesFromFields r rOffset fieldInfos - let rNew := mkResultUniverse us rOffset (isPropCandidate fieldInfos) - assignLevelMVar mvarId rNew - instantiateMVars type - | _ => throwError "failed to compute resulting universe level of structure, provide universe explicitly" + unless r.isMVar do + throwError "failed to compute resulting universe level of inductive datatype, provide universe explicitly: {r}" + let us ← collectUniversesFromFields r rOffset fieldInfos + trace[Elab.structure] "updateResultingUniverse us: {us}, r: {r}, rOffset: {rOffset}" + let rNew := mkResultUniverse us rOffset (isPropCandidate fieldInfos) + assignLevelMVar r.mvarId! rNew + instantiateMVars type private def collectLevelParamsInFVar (s : CollectLevelParams.State) (fvar : Expr) : TermElabM CollectLevelParams.State := do let type ← inferType fvar @@ -704,9 +771,13 @@ private def mkCtor (view : StructView) (levelParams : List Name) (params : Array @[extern "lean_mk_projections"] private opaque mkProjections (env : Environment) (structName : Name) (projs : List Name) (isClass : Bool) : Except KernelException Environment -private def addProjections (structName : Name) (projs : List Name) (isClass : Bool) : TermElabM Unit := do +private def addProjections (r : ElabStructHeaderResult) (fieldInfos : Array StructFieldInfo) : TermElabM Unit := do + if r.type.isProp then + if let some fieldInfo ← fieldInfos.findM? fun fieldInfo => not <$> Meta.isProof fieldInfo.fvar then + throwErrorAt fieldInfo.ref m!"failed to generate projections for 'Prop' structure, field '{format fieldInfo.name}' is not a proof" + let projNames := (fieldInfos.filter fun (info : StructFieldInfo) => !info.isFromParent).toList.map fun (info : StructFieldInfo) => info.declName let env ← getEnv - let env ← ofExceptKernelException (mkProjections env structName projs isClass) + let env ← ofExceptKernelException (mkProjections env r.view.declName projNames r.view.isClass) setEnv env private def registerStructure (structName : Name) (infos : Array StructFieldInfo) : TermElabM Unit := do @@ -735,25 +806,28 @@ private def registerStructure (structName : Name) (infos : Array StructFieldInfo private def mkAuxConstructions (declName : Name) : TermElabM Unit := do let env ← getEnv - let hasUnit := env.contains `PUnit - let hasEq := env.contains `Eq - let hasHEq := env.contains `HEq + let hasEq := env.contains ``Eq + let hasHEq := env.contains ``HEq + let hasUnit := env.contains ``PUnit mkRecOn declName if hasUnit then mkCasesOn declName if hasUnit && hasEq && hasHEq then mkNoConfusion declName -private def addDefaults (lctx : LocalContext) (defaultAuxDecls : Array (Name × Expr × Expr)) : TermElabM Unit := do - let localInsts ← getLocalInstances - withLCtx lctx localInsts do - defaultAuxDecls.forM fun (declName, type, value) => do - let value ← instantiateMVars value - if value.hasExprMVar then - throwError "invalid default value for field, it contains metavariables{indentExpr value}" - /- The identity function is used as "marker". -/ - let value ← mkId value - -- No need to compile the definition, since it is only used during elaboration. - discard <| mkAuxDefinition declName type value (zetaDelta := true) (compile := false) - setReducibleAttribute declName +private def addDefaults (lctx : LocalContext) (fieldInfos : Array StructFieldInfo) : TermElabM Unit := do + withLCtx lctx (← getLocalInstances) do + fieldInfos.forM fun fieldInfo => do + if let some value := fieldInfo.value? then + let declName := mkDefaultFnOfProjFn fieldInfo.declName + let type ← inferType fieldInfo.fvar + let value ← instantiateMVars value + if value.hasExprMVar then + discard <| Term.logUnassignedUsingErrorInfos (← getMVars value) + throwErrorAt fieldInfo.ref "invalid default value for field '{format fieldInfo.name}', it contains metavariables{indentExpr value}" + /- The identity function is used as "marker". -/ + let value ← mkId value + -- No need to compile the definition, since it is only used during elaboration. + discard <| mkAuxDefinition declName type value (zetaDelta := true) (compile := false) + setReducibleAttribute declName /-- Given `type` of the form `forall ... (source : A), B`, return `forall ... [source : A], B`. @@ -767,12 +841,11 @@ private def setSourceInstImplicit (type : Expr) : Expr := type.updateForall! .instImplicit d b | _ => unreachable! -private partial def mkCoercionToCopiedParent (levelParams : List Name) (params : Array Expr) (view : StructView) (parentType : Expr) : MetaM Unit := do +private partial def mkCoercionToCopiedParent (levelParams : List Name) (params : Array Expr) (view : StructView) (parentStructName : Name) (parentType : Expr) : MetaM Unit := do let env ← getEnv let structName := view.declName let sourceFieldNames := getStructureFieldsFlattened env structName let structType := mkAppN (Lean.mkConst structName (levelParams.map mkLevelParam)) params - let Expr.const parentStructName _ ← pure parentType.getAppFn | unreachable! let binfo := if view.isClass && isClass env parentStructName then BinderInfo.instImplicit else BinderInfo.default withLocalDeclD `self structType fun source => do let mut declType ← instantiateMVars (← mkForallFVars params (← mkForallFVars #[source] parentType)) @@ -811,137 +884,156 @@ private partial def mkCoercionToCopiedParent (levelParams : List Name) (params : else setReducibleAttribute declName -private def elabStructureView (view : StructView) : TermElabM Unit := do - view.fields.forM fun field => do - if field.declName == view.ctor.declName then - throwErrorAt field.ref "invalid field name '{field.name}', it is equal to structure constructor name" - addAuxDeclarationRanges field.declName field.ref field.ref - let type ← Term.elabType view.type - unless validStructType type do throwErrorAt view.type "expected Type" - withRef view.ref do - withParents view fun fieldInfos copiedParents => do - withFields view.fields fieldInfos fun fieldInfos => do +private def elabStructHeader (view : StructView) : TermElabM ElabStructHeaderResult := + Term.withAutoBoundImplicitForbiddenPred (fun n => view.shortDeclName == n) do + Term.withAutoBoundImplicit do + Term.elabBinders view.binders.getArgs fun params => do + elabParents view fun parentFieldInfos parents => do + let type ← Term.elabType view.type Term.synthesizeSyntheticMVarsNoPostponing - let u ← getResultUniverse type - let univToInfer? ← shouldInferResultUniverse u - withUsed view.scopeVars view.params fieldInfos fun scopeVars => do - let fieldInfos ← levelMVarToParam scopeVars view.params fieldInfos univToInfer? - let type ← withRef view.ref do - if univToInfer?.isSome then - updateResultingUniverse fieldInfos type - else - checkResultingUniverse (← getResultUniverse type) - pure type - trace[Elab.structure] "type: {type}" - let usedLevelNames ← collectLevelParamsInStructure type scopeVars view.params fieldInfos - match sortDeclLevelParams view.scopeLevelNames view.allUserLevelNames usedLevelNames with - | Except.error msg => withRef view.ref <| throwError msg - | Except.ok levelParams => - let params := scopeVars ++ view.params - let ctor ← mkCtor view levelParams params fieldInfos - let type ← mkForallFVars params type - let type ← instantiateMVars type - let indType := { name := view.declName, type := type, ctors := [ctor] : InductiveType } - let decl := Declaration.inductDecl levelParams params.size [indType] view.modifiers.isUnsafe - Term.ensureNoUnassignedMVars decl - addDecl decl - let projNames := (fieldInfos.filter fun (info : StructFieldInfo) => !info.isFromParent).toList.map fun (info : StructFieldInfo) => info.declName - addProjections view.declName projNames view.isClass - registerStructure view.declName fieldInfos - mkAuxConstructions view.declName - let instParents ← fieldInfos.filterM fun info => do - let decl ← Term.getFVarLocalDecl! info.fvar - pure (info.isSubobject && decl.binderInfo.isInstImplicit) - withSaveInfoContext do -- save new env - Term.addLocalVarInfo view.ref[1] (← mkConstWithLevelParams view.declName) - if let some _ := view.ctor.ref.getPos? (canonicalOnly := true) then - Term.addTermInfo' view.ctor.ref (← mkConstWithLevelParams view.ctor.declName) (isBinder := true) - for field in view.fields do - -- may not exist if overriding inherited field - if (← getEnv).contains field.declName then - Term.addTermInfo' field.ref (← mkConstWithLevelParams field.declName) (isBinder := true) - Term.applyAttributesAt view.declName view.modifiers.attrs AttributeApplicationTime.afterTypeChecking - let projInstances := instParents.toList.map fun info => info.declName - projInstances.forM fun declName => addInstance declName AttributeKind.global (eval_prio default) - copiedParents.forM fun parent => mkCoercionToCopiedParent levelParams params view parent - let lctx ← getLCtx - let fieldsWithDefault := fieldInfos.filter fun info => info.value?.isSome - let defaultAuxDecls ← fieldsWithDefault.mapM fun info => do - let type ← inferType info.fvar - pure (mkDefaultFnOfProjFn info.declName, type, info.value?.get!) - /- The `lctx` and `defaultAuxDecls` are used to create the auxiliary "default value" declarations - The parameters `params` for these definitions must be marked as implicit, and all others as explicit. -/ - let lctx := - params.foldl (init := lctx) fun (lctx : LocalContext) (p : Expr) => - if p.isFVar then - lctx.setBinderInfo p.fvarId! BinderInfo.implicit - else - lctx - let lctx := - fieldInfos.foldl (init := lctx) fun (lctx : LocalContext) (info : StructFieldInfo) => - if info.isFromParent then lctx -- `fromParent` fields are elaborated as let-decls, and are zeta-expanded when creating "default value" auxiliary functions - else lctx.setBinderInfo info.fvar.fvarId! BinderInfo.default - addDefaults lctx defaultAuxDecls - -/- -leading_parser (structureTk <|> classTk) >> declId >> many Term.bracketedBinder >> optional «extends» >> Term.optType >> - optional (("where" <|> ":=") >> optional structCtor >> structFields) >> optDeriving - -where -def «extends» := leading_parser " extends " >> sepBy1 termParser ", " -def typeSpec := leading_parser " : " >> termParser -def optType : Parser := optional typeSpec + let u ← mkFreshLevelMVar + unless ← isDefEq type (mkSort u) do + throwErrorAt view.type "invalid structure type, expecting 'Type _' or 'Prop'" + let type ← instantiateMVars (← whnf type) + Term.addAutoBoundImplicits' params type fun params type => do + let levelNames ← Term.getLevelNames + trace[Elab.structure] "header params: {params}, type: {type}, levelNames: {levelNames}" + return { lctx := (← getLCtx), localInsts := (← getLocalInstances), levelNames, params, type, view, parents, parentFieldInfos } + +private def mkTypeFor (r : ElabStructHeaderResult) : TermElabM Expr := do + withLCtx r.lctx r.localInsts do + mkForallFVars r.params r.type -def structFields := leading_parser many (structExplicitBinder <|> structImplicitBinder <|> structInstBinder) -def structCtor := leading_parser try (declModifiers >> ident >> " :: ") +/-- +Create a local declaration for the structure and execute `x params indFVar`, where `params` are the structure's type parameters and +`indFVar` is the new local declaration. +-/ +private partial def withStructureLocalDecl (r : ElabStructHeaderResult) (x : Array Expr → Expr → TermElabM α) : TermElabM α := do + let declName := r.view.declName + let shortDeclName := r.view.shortDeclName + let type ← mkTypeFor r + let params := r.params + withLCtx r.lctx r.localInsts <| withRef r.view.ref do + Term.withAuxDecl shortDeclName type declName fun indFVar => + x params indFVar +/-- +Remark: `numVars <= numParams`. +`numVars` is the number of context `variables` used in the declaration, +and `numParams - numVars` is the number of parameters provided as binders in the declaration. -/ +private def mkInductiveType (view : StructView) (indFVar : Expr) (levelNames : List Name) + (numVars : Nat) (numParams : Nat) (type : Expr) (ctor : Constructor) : TermElabM InductiveType := do + let levelParams := levelNames.map mkLevelParam + let const := mkConst view.declName levelParams + let ctorType ← forallBoundedTelescope ctor.type numParams fun params type => do + if type.containsFVar indFVar.fvarId! then + throwErrorAt view.ref "Recursive structures are not yet supported." + let type := type.replace fun e => + if e == indFVar then + mkAppN const (params.extract 0 numVars) + else + none + instantiateMVars (← mkForallFVars params type) + return { name := view.declName, type := ← instantiateMVars type, ctors := [{ ctor with type := ← instantiateMVars ctorType }] } + +def mkStructureDecl (vars : Array Expr) (view : StructView) : TermElabM Unit := Term.withoutSavingRecAppSyntax do + let scopeLevelNames ← Term.getLevelNames + let isUnsafe := view.modifiers.isUnsafe + withRef view.ref <| Term.withLevelNames view.levelNames do + let r ← elabStructHeader view + Term.synthesizeSyntheticMVarsNoPostponing + withLCtx r.lctx r.localInsts do + withStructureLocalDecl r fun params indFVar => do + trace[Elab.structure] "indFVar: {indFVar}" + Term.addLocalVarInfo view.declId indFVar + withFields view.fields r.parentFieldInfos fun fieldInfos => + withRef view.ref do + Term.synthesizeSyntheticMVarsNoPostponing + let type ← instantiateMVars r.type + let u ← getResultUniverse type + let univToInfer? ← shouldInferResultUniverse u + withUsed vars params fieldInfos fun scopeVars => do + let fieldInfos ← levelMVarToParam scopeVars params fieldInfos univToInfer? + let type ← withRef view.ref do + if univToInfer?.isSome then + updateResultingUniverse fieldInfos type + else + checkResultingUniverse (← getResultUniverse type) + pure type + trace[Elab.structure] "type: {type}" + let usedLevelNames ← collectLevelParamsInStructure type scopeVars params fieldInfos + match sortDeclLevelParams scopeLevelNames r.levelNames usedLevelNames with + | Except.error msg => throwErrorAt view.declId msg + | Except.ok levelParams => + let params := scopeVars ++ params + let ctor ← mkCtor view levelParams params fieldInfos + let type ← mkForallFVars params type + let type ← instantiateMVars type + let indType ← mkInductiveType view indFVar levelParams scopeVars.size params.size type ctor + let decl := Declaration.inductDecl levelParams params.size [indType] isUnsafe + Term.ensureNoUnassignedMVars decl + addDecl decl + -- rename indFVar so that it does not shadow the actual declaration: + let lctx := (← getLCtx).modifyLocalDecl indFVar.fvarId! fun decl => decl.setUserName .anonymous + withLCtx lctx (← getLocalInstances) do + addProjections r fieldInfos + registerStructure view.declName fieldInfos + mkAuxConstructions view.declName + let instParents ← fieldInfos.filterM fun info => do + let decl ← Term.getFVarLocalDecl! info.fvar + pure (info.isSubobject && decl.binderInfo.isInstImplicit) + withSaveInfoContext do -- save new env + Term.addLocalVarInfo view.ref[1] (← mkConstWithLevelParams view.declName) + if let some _ := view.ctor.ref.getPos? (canonicalOnly := true) then + Term.addTermInfo' view.ctor.ref (← mkConstWithLevelParams view.ctor.declName) (isBinder := true) + for field in view.fields do + -- may not exist if overriding inherited field + if (← getEnv).contains field.declName then + Term.addTermInfo' field.ref (← mkConstWithLevelParams field.declName) (isBinder := true) + withRef view.declId do + Term.applyAttributesAt view.declName view.modifiers.attrs AttributeApplicationTime.afterTypeChecking + let projInstances := instParents.toList.map fun info => info.declName + projInstances.forM fun declName => addInstance declName AttributeKind.global (eval_prio default) + r.parents.forM fun parent => do + if !parent.subobject then + mkCoercionToCopiedParent levelParams params view parent.structName parent.type + let lctx ← getLCtx + /- The `lctx` and `defaultAuxDecls` are used to create the auxiliary "default value" declarations + The parameters `params` for these definitions must be marked as implicit, and all others as explicit. -/ + let lctx := + params.foldl (init := lctx) fun (lctx : LocalContext) (p : Expr) => + if p.isFVar then + lctx.setBinderInfo p.fvarId! BinderInfo.implicit + else + lctx + let lctx := + fieldInfos.foldl (init := lctx) fun (lctx : LocalContext) (info : StructFieldInfo) => + if info.isFromParent then lctx -- `fromParent` fields are elaborated as let-decls, and are zeta-expanded when creating "default value" auxiliary functions + else lctx.setBinderInfo info.fvar.fvarId! BinderInfo.default + addDefaults lctx fieldInfos + + +def elabStructureView (vars : Array Expr) (view : StructView) : TermElabM Unit := do + Term.withDeclName view.declName <| withRef view.ref do + mkStructureDecl vars view + unless view.isClass do + Lean.Meta.IndPredBelow.mkBelow view.declName + mkSizeOfInstances view.declName + mkInjectiveTheorems view.declName + +def elabStructureViewPostprocessing (view : StructView) : CommandElabM Unit := do + view.derivingClasses.forM fun classView => classView.applyHandlers #[view.declName] + runTermElabM fun _ => Term.withDeclName view.declName <| withRef view.declId do + Term.applyAttributesAt view.declName view.modifiers.attrs .afterCompilation + def elabStructure (modifiers : Modifiers) (stx : Syntax) : CommandElabM Unit := do - checkValidInductiveModifier modifiers - let isClass := stx[0].getKind == ``Parser.Command.classTk - let modifiers := if isClass then modifiers.addAttr { name := `class } else modifiers - let declId := stx[1] - let params := stx[2].getArgs - let exts := stx[3] - let parents := if exts.isNone then #[] else exts[0][1].getSepArgs - let optType := stx[4] - let derivingClassViews ← liftCoreM <| getOptDerivingClasses stx[6] - let type ← if optType.isNone then `(Sort _) else pure optType[0][1] - let declName ← - runTermElabM fun scopeVars => do - let scopeLevelNames ← Term.getLevelNames - let ⟨name, declName, allUserLevelNames⟩ ← Elab.expandDeclId (← getCurrNamespace) scopeLevelNames declId modifiers - Term.withAutoBoundImplicitForbiddenPred (fun n => name == n) do - addDeclarationRanges declName modifiers.stx stx - Term.withDeclName declName do - let ctor ← expandCtor stx modifiers declName - let fields ← expandFields stx modifiers declName - Term.withLevelNames allUserLevelNames <| Term.withAutoBoundImplicit <| - Term.elabBinders params fun params => do - Term.synthesizeSyntheticMVarsNoPostponing - let params ← Term.addAutoBoundImplicits params - let allUserLevelNames ← Term.getLevelNames - elabStructureView { - ref := stx - modifiers - scopeLevelNames - allUserLevelNames - declName - isClass - scopeVars - params - parents - type - ctor - fields - } - unless isClass do - mkSizeOfInstances declName - mkInjectiveTheorems declName - return declName - derivingClassViews.forM fun view => view.applyHandlers #[declName] - runTermElabM fun _ => Term.withDeclName declName do - Term.applyAttributesAt declName modifiers.attrs .afterCompilation + let view ← runTermElabM fun vars => do + let view ← structureSyntaxToView modifiers stx + trace[Elab.structure] "view.levelNames: {view.levelNames}" + elabStructureView vars view + pure view + elabStructureViewPostprocessing view builtin_initialize registerTraceClass `Elab.structure diff --git a/src/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/Reflect.lean b/src/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/Reflect.lean index f156cdac4f2a..7a1395adfd14 100644 --- a/src/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/Reflect.lean +++ b/src/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/Reflect.lean @@ -29,6 +29,7 @@ instance : ToExpr BVBinOp where | .mul => mkConst ``BVBinOp.mul | .udiv => mkConst ``BVBinOp.udiv | .umod => mkConst ``BVBinOp.umod + | .sdiv => mkConst ``BVBinOp.sdiv toTypeExpr := mkConst ``BVBinOp instance : ToExpr BVUnOp where diff --git a/src/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/ReifiedBVExpr.lean b/src/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/ReifiedBVExpr.lean index 3df04f164842..64c2f9552de7 100644 --- a/src/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/ReifiedBVExpr.lean +++ b/src/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/ReifiedBVExpr.lean @@ -102,6 +102,8 @@ where binaryReflection lhsExpr rhsExpr .udiv ``Std.Tactic.BVDecide.Reflect.BitVec.udiv_congr | HMod.hMod _ _ _ _ lhsExpr rhsExpr => binaryReflection lhsExpr rhsExpr .umod ``Std.Tactic.BVDecide.Reflect.BitVec.umod_congr + | BitVec.sdiv _ lhsExpr rhsExpr => + binaryReflection lhsExpr rhsExpr .sdiv ``Std.Tactic.BVDecide.Reflect.BitVec.sdiv_congr | Complement.complement _ _ innerExpr => unaryReflection innerExpr .not ``Std.Tactic.BVDecide.Reflect.BitVec.not_congr | HShiftLeft.hShiftLeft _ β _ _ innerExpr distanceExpr => diff --git a/src/Lean/Elab/Tactic/Conv/Unfold.lean b/src/Lean/Elab/Tactic/Conv/Unfold.lean index aa791a4d38e6..2bbc9439c2db 100644 --- a/src/Lean/Elab/Tactic/Conv/Unfold.lean +++ b/src/Lean/Elab/Tactic/Conv/Unfold.lean @@ -12,13 +12,16 @@ open Meta @[builtin_tactic Lean.Parser.Tactic.Conv.unfold] def evalUnfold : Tactic := fun stx => withMainContext do for declNameId in stx[1].getArgs do - let e ← elabTermForApply declNameId (mayPostpone := false) - match e with - | .const declName _ => - applySimpResult (← unfold (← getLhs) declName) - | .fvar declFVarId => - let lhs ← instantiateMVars (← getLhs) - changeLhs (← Meta.zetaDeltaFVars lhs #[declFVarId]) - | _ => throwErrorAt declNameId m!"'unfold' conv tactic failed, expression {e} is not a global or local constant" + withRef declNameId do + let e ← elabTermForApply declNameId (mayPostpone := false) + match e with + | .const declName _ => + applySimpResult (← unfold (← getLhs) declName) + | .fvar declFVarId => + unless ← declFVarId.isLetVar do + throwError "conv tactic 'unfold' failed, local variable '{Expr.fvar declFVarId}' has no definition" + let lhs ← instantiateMVars (← getLhs) + changeLhs (← Meta.zetaDeltaFVars lhs #[declFVarId]) + | _ => throwError "conv tactic 'unfold' failed, expression {e} is not a global or local constant" end Lean.Elab.Tactic.Conv diff --git a/src/Lean/Elab/Tactic/Ext.lean b/src/Lean/Elab/Tactic/Ext.lean index dbfe47f4663d..d8011ad50351 100644 --- a/src/Lean/Elab/Tactic/Ext.lean +++ b/src/Lean/Elab/Tactic/Ext.lean @@ -123,7 +123,7 @@ def realizeExtTheorem (structName : Name) (flat : Bool) : Elab.Command.CommandEl levelParams := info.levelParams } modifyEnv fun env => addProtected env extName - addAuxDeclarationRanges extName (← getRef) (← getRef) + addDeclarationRangesFromSyntax extName (← getRef) catch e => throwError m!"\ Failed to generate an 'ext' theorem for '{MessageData.ofConstName structName}': {e.toMessageData}" @@ -161,7 +161,7 @@ def realizeExtIffTheorem (extName : Name) : Elab.Command.CommandElabM Name := do -- Only declarations in a namespace can be protected: unless extIffName.isAtomic do modifyEnv fun env => addProtected env extIffName - addAuxDeclarationRanges extName (← getRef) (← getRef) + addDeclarationRangesFromSyntax extName (← getRef) catch e => throwError m!"\ Failed to generate an 'ext_iff' theorem from '{MessageData.ofConstName extName}': {e.toMessageData}\n\ diff --git a/src/Lean/Elab/Tactic/Generalize.lean b/src/Lean/Elab/Tactic/Generalize.lean index 3860107a687b..c76a4a048e55 100644 --- a/src/Lean/Elab/Tactic/Generalize.lean +++ b/src/Lean/Elab/Tactic/Generalize.lean @@ -30,7 +30,7 @@ open Meta args := args.push { hName?, expr, xName? := arg[3].getId : GeneralizeArg } let hyps ← match expandOptLocation stx[2] with | .targets hyps _ => getFVarIds hyps - | .wildcard => pure (← getLCtx).getFVarIds + | .wildcard => pure ((← getLocalHyps).map (·.fvarId!)) let mvarId ← getMainGoal mvarId.withContext do let (_, newVars, mvarId) ← mvarId.generalizeHyp args hyps diff --git a/src/Lean/Elab/Tactic/Unfold.lean b/src/Lean/Elab/Tactic/Unfold.lean index 7e77caa3244d..0bae5e82b89e 100644 --- a/src/Lean/Elab/Tactic/Unfold.lean +++ b/src/Lean/Elab/Tactic/Unfold.lean @@ -29,13 +29,15 @@ def zetaDeltaTarget (declFVarId : FVarId) : TacticM Unit := do for declNameId in stx[1].getArgs do go declNameId loc where - go (declNameId : Syntax) (loc : Location) : TacticM Unit := withMainContext do + go (declNameId : Syntax) (loc : Location) : TacticM Unit := withMainContext <| withRef declNameId do let e ← elabTermForApply declNameId (mayPostpone := false) match e with | .const declName _ => withLocation loc (unfoldLocalDecl declName) (unfoldTarget declName) (throwTacticEx `unfold · m!"did not unfold '{declName}'") | .fvar declFVarId => + unless ← declFVarId.isLetVar do + throwError "tactic 'unfold' failed, local variable '{Expr.fvar declFVarId}' has no definition" withLocation loc (zetaDeltaLocalDecl declFVarId) (zetaDeltaTarget declFVarId) (throwTacticEx `unfold · m!"did not unfold '{e}'") - | _ => withRef declNameId <| throwTacticEx `unfold (← getMainGoal) m!"expression {e} is not a global or local constant" + | _ => throwTacticEx `unfold (← getMainGoal) m!"expression {e} is not a global or local constant" end Lean.Elab.Tactic diff --git a/src/Lean/Language/Lean.lean b/src/Lean/Language/Lean.lean index 1db498894694..83a685d2a8e4 100644 --- a/src/Lean/Language/Lean.lean +++ b/src/Lean/Language/Lean.lean @@ -300,7 +300,9 @@ General notes: * We must make sure to trigger `oldCancelTk?` as soon as discarding `old?`. * Control flow up to finding the last still-valid snapshot (which should be quick) is synchronous so as not to report this "fast forwarding" to the user as well as to make sure the next run sees all - fast-forwarded snapshots without having to wait on tasks. + fast-forwarded snapshots without having to wait on tasks. It also ensures this part cannot be + delayed by threadpool starvation. We track whether we are still on the fast-forwarding path using + the `sync` parameter on `parseCmd` and spawn an elaboration task when we leave it. -/ partial def process (setupImports : Syntax → ProcessingT IO (Except HeaderProcessedSnapshot SetupImportsResult)) @@ -330,7 +332,7 @@ where -- elaboration reuse oldProcSuccess.firstCmdSnap.bindIO (sync := true) fun oldCmd => do let prom ← IO.Promise.new - let _ ← IO.asTask (parseCmd oldCmd newParserState oldProcSuccess.cmdState prom ctx) + parseCmd oldCmd newParserState oldProcSuccess.cmdState prom (sync := true) ctx return .pure { diagnostics := oldProcessed.diagnostics result? := some { @@ -446,7 +448,7 @@ where let parserState := Runtime.markPersistent parserState let cmdState := Runtime.markPersistent cmdState let ctx := Runtime.markPersistent ctx - let _ ← IO.asTask (parseCmd none parserState cmdState prom ctx) + parseCmd none parserState cmdState prom (sync := true) ctx return { diagnostics infoTree? := cmdState.infoState.trees[0]! @@ -457,24 +459,10 @@ where } parseCmd (old? : Option CommandParsedSnapshot) (parserState : Parser.ModuleParserState) - (cmdState : Command.State) (prom : IO.Promise CommandParsedSnapshot) : + (cmdState : Command.State) (prom : IO.Promise CommandParsedSnapshot) (sync : Bool) : LeanProcessingM Unit := do let ctx ← read - -- check for cancellation, most likely during elaboration of previous command, before starting - -- processing of next command - if (← ctx.newCancelTk.isSet) then - -- this is a bit ugly as we don't want to adjust our API with `Option`s just for cancellation - -- (as no-one should look at this result in that case) but anything containing `Environment` - -- is not `Inhabited` - prom.resolve <| .mk (nextCmdSnap? := none) { - diagnostics := .empty, stx := .missing, parserState - elabSnap := .pure <| .ofTyped { diagnostics := .empty : SnapshotLeaf } - finishedSnap := .pure { diagnostics := .empty, cmdState } - tacticCache := (← IO.mkRef {}) - } - return - let unchanged old newParserState : BaseIO Unit := -- when syntax is unchanged, reuse command processing task as is -- NOTE: even if the syntax tree is functionally unchanged, the new parser state may still @@ -482,11 +470,11 @@ where -- from `old` if let some oldNext := old.nextCmdSnap? then do let newProm ← IO.Promise.new - let _ ← old.data.finishedSnap.bindIO fun oldFinished => + let _ ← old.data.finishedSnap.bindIO (sync := true) fun oldFinished => -- also wait on old command parse snapshot as parsing is cheap and may allow for -- elaboration reuse oldNext.bindIO (sync := true) fun oldNext => do - parseCmd oldNext newParserState oldFinished.cmdState newProm ctx + parseCmd oldNext newParserState oldFinished.cmdState newProm sync ctx return .pure () prom.resolve <| .mk (data := old.data) (nextCmdSnap? := some { range? := none, task := newProm.result }) else prom.resolve old -- terminal command, we're done! @@ -521,44 +509,61 @@ where if let some tk := ctx.oldCancelTk? then tk.set - -- definitely resolved in `doElab` task - let elabPromise ← IO.Promise.new - let finishedPromise ← IO.Promise.new - -- (Try to) use last line of command as range for final snapshot task. This ensures we do not - -- retract the progress bar to a previous position in case the command support incremental - -- reporting but has significant work after resolving its last incremental promise, such as - -- final type checking; if it does not support incrementality, `elabSnap` constructed in - -- `parseCmd` and containing the entire range of the command will determine the reported - -- progress and be resolved effectively at the same time as this snapshot task, so `tailPos` is - -- irrelevant in this case. - let endRange? := stx.getTailPos?.map fun pos => ⟨pos, pos⟩ - let finishedSnap := { range? := endRange?, task := finishedPromise.result } - let tacticCache ← old?.map (·.data.tacticCache) |>.getDM (IO.mkRef {}) - - let minimalSnapshots := internal.cmdlineSnapshots.get cmdState.scopes.head!.opts - let next? ← if Parser.isTerminalCommand stx then pure none - -- for now, wait on "command finished" snapshot before parsing next command - else some <$> IO.Promise.new - let diagnostics ← Snapshot.Diagnostics.ofMessageLog msgLog - let data := if minimalSnapshots && !Parser.isTerminalCommand stx then { - diagnostics - stx := .missing - parserState := {} - elabSnap := { range? := stx.getRange?, task := elabPromise.result } - finishedSnap - tacticCache - } else { - diagnostics, stx, parserState, tacticCache - elabSnap := { range? := stx.getRange?, task := elabPromise.result } - finishedSnap - } - prom.resolve <| .mk (nextCmdSnap? := next?.map - ({ range? := some ⟨parserState.pos, ctx.input.endPos⟩, task := ·.result })) data - let cmdState ← doElab stx cmdState beginPos - { old? := old?.map fun old => ⟨old.data.stx, old.data.elabSnap⟩, new := elabPromise } - finishedPromise tacticCache ctx - if let some next := next? then - parseCmd none parserState cmdState next ctx + -- check for cancellation, most likely during elaboration of previous command, before starting + -- processing of next command + if (← ctx.newCancelTk.isSet) then + -- this is a bit ugly as we don't want to adjust our API with `Option`s just for cancellation + -- (as no-one should look at this result in that case) but anything containing `Environment` + -- is not `Inhabited` + prom.resolve <| .mk (nextCmdSnap? := none) { + diagnostics := .empty, stx := .missing, parserState + elabSnap := .pure <| .ofTyped { diagnostics := .empty : SnapshotLeaf } + finishedSnap := .pure { diagnostics := .empty, cmdState } + tacticCache := (← IO.mkRef {}) + } + return + + -- Start new task when leaving fast-forwarding path; see "General notes" above + let _ ← (if sync then BaseIO.asTask else (.pure <$> ·)) do + -- definitely resolved in `doElab` task + let elabPromise ← IO.Promise.new + let finishedPromise ← IO.Promise.new + -- (Try to) use last line of command as range for final snapshot task. This ensures we do not + -- retract the progress bar to a previous position in case the command support incremental + -- reporting but has significant work after resolving its last incremental promise, such as + -- final type checking; if it does not support incrementality, `elabSnap` constructed in + -- `parseCmd` and containing the entire range of the command will determine the reported + -- progress and be resolved effectively at the same time as this snapshot task, so `tailPos` is + -- irrelevant in this case. + let endRange? := stx.getTailPos?.map fun pos => ⟨pos, pos⟩ + let finishedSnap := { range? := endRange?, task := finishedPromise.result } + let tacticCache ← old?.map (·.data.tacticCache) |>.getDM (IO.mkRef {}) + + let minimalSnapshots := internal.cmdlineSnapshots.get cmdState.scopes.head!.opts + let next? ← if Parser.isTerminalCommand stx then pure none + -- for now, wait on "command finished" snapshot before parsing next command + else some <$> IO.Promise.new + let diagnostics ← Snapshot.Diagnostics.ofMessageLog msgLog + let data := if minimalSnapshots && !Parser.isTerminalCommand stx then { + diagnostics + stx := .missing + parserState := {} + elabSnap := { range? := stx.getRange?, task := elabPromise.result } + finishedSnap + tacticCache + } else { + diagnostics, stx, parserState, tacticCache + elabSnap := { range? := stx.getRange?, task := elabPromise.result } + finishedSnap + } + prom.resolve <| .mk (nextCmdSnap? := next?.map + ({ range? := some ⟨parserState.pos, ctx.input.endPos⟩, task := ·.result })) data + let cmdState ← doElab stx cmdState beginPos + { old? := old?.map fun old => ⟨old.data.stx, old.data.elabSnap⟩, new := elabPromise } + finishedPromise tacticCache ctx + if let some next := next? then + -- We're definitely off the fast-forwarding path now + parseCmd none parserState cmdState next (sync := false) ctx doElab (stx : Syntax) (cmdState : Command.State) (beginPos : String.Pos) (snap : SnapshotBundle DynamicSnapshot) (finishedPromise : IO.Promise CommandFinishedSnapshot) @@ -625,7 +630,7 @@ def processCommands (inputCtx : Parser.InputContext) (parserState : Parser.Modul (old? : Option (Parser.InputContext × CommandParsedSnapshot) := none) : BaseIO (Task CommandParsedSnapshot) := do let prom ← IO.Promise.new - process.parseCmd (old?.map (·.2)) parserState commandState prom + process.parseCmd (old?.map (·.2)) parserState commandState prom (sync := true) |>.run (old?.map (·.1)) |>.run { inputCtx with } return prom.result diff --git a/src/Lean/Meta/AppBuilder.lean b/src/Lean/Meta/AppBuilder.lean index 57f125b388a7..8a58c903b88b 100644 --- a/src/Lean/Meta/AppBuilder.lean +++ b/src/Lean/Meta/AppBuilder.lean @@ -28,6 +28,7 @@ def mkExpectedTypeHint (e : Expr) (expectedType : Expr) : MetaM Expr := do /-- `mkLetFun x v e` creates the encoding for the `let_fun x := v; e` expression. The expression `x` can either be a free variable or a metavariable, and the function suitably abstracts `x` in `e`. +NB: `x` must not be a let-bound free variable. -/ def mkLetFun (x : Expr) (v : Expr) (e : Expr) : MetaM Expr := do let f ← mkLambdaFVars #[x] e diff --git a/src/Lean/Meta/DiscrTree.lean b/src/Lean/Meta/DiscrTree.lean index ad1ec8021260..79d2bff9f7e5 100644 --- a/src/Lean/Meta/DiscrTree.lean +++ b/src/Lean/Meta/DiscrTree.lean @@ -767,9 +767,6 @@ where namespace Trie --- `Inhabited` instance to allow `partial` definitions below. -private local instance [Monad m] : Inhabited (σ → β → m σ) := ⟨fun s _ => pure s⟩ - /-- Monadically fold the keys and values stored in a `Trie`. -/ diff --git a/src/Lean/Meta/LitValues.lean b/src/Lean/Meta/LitValues.lean index 19b8efe3783a..0bc7acd03a21 100644 --- a/src/Lean/Meta/LitValues.lean +++ b/src/Lean/Meta/LitValues.lean @@ -5,6 +5,7 @@ Authors: Leonardo de Moura -/ prelude import Lean.Meta.Basic +import Init.Control.Option namespace Lean.Meta diff --git a/src/Lean/Meta/Offset.lean b/src/Lean/Meta/Offset.lean index eac7e1a55c6c..01216f454284 100644 --- a/src/Lean/Meta/Offset.lean +++ b/src/Lean/Meta/Offset.lean @@ -4,6 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE. Authors: Leonardo de Moura -/ prelude +import Init.Control.Option import Lean.Data.LBool import Lean.Meta.InferType import Lean.Meta.NatInstTesters diff --git a/src/Lean/Meta/Tactic/FunInd.lean b/src/Lean/Meta/Tactic/FunInd.lean index 15da6fef3200..19c167ec70d9 100644 --- a/src/Lean/Meta/Tactic/FunInd.lean +++ b/src/Lean/Meta/Tactic/FunInd.lean @@ -262,8 +262,8 @@ partial def foldAndCollect (oldIH newIH : FVarId) (isRecCall : Expr → Option E if let some (n, t, v, b) := e.letFun? then let t' ← foldAndCollect oldIH newIH isRecCall t let v' ← foldAndCollect oldIH newIH isRecCall v - return ← withLetDecl n t' v' fun x => do - M.localMapM (mkLetFVars (usedLetOnly := true) #[x] ·) do + return ← withLocalDeclD n t' fun x => do + M.localMapM (mkLetFun x v' ·) do let b' ← foldAndCollect oldIH newIH isRecCall (b.instantiate1 x) mkLetFun x v' b' @@ -598,6 +598,11 @@ partial def buildInductionBody (toClear : Array FVarId) (goal : Expr) buildInductionBody toClear expAltType oldIH newIH isRecCall alt) return matcherApp'.toExpr + -- we look through mdata + if e.isMData then + let b ← buildInductionBody toClear goal oldIH newIH isRecCall e.mdataExpr! + return e.updateMData! b + if let .letE n t v b _ := e then let t' ← foldAndCollect oldIH newIH isRecCall t let v' ← foldAndCollect oldIH newIH isRecCall v @@ -608,7 +613,7 @@ partial def buildInductionBody (toClear : Array FVarId) (goal : Expr) if let some (n, t, v, b) := e.letFun? then let t' ← foldAndCollect oldIH newIH isRecCall t let v' ← foldAndCollect oldIH newIH isRecCall v - return ← withLocalDecl n .default t' fun x => M2.branch do + return ← withLocalDeclD n t' fun x => M2.branch do let b' ← buildInductionBody toClear goal oldIH newIH isRecCall (b.instantiate1 x) mkLetFun x v' b' diff --git a/src/Lean/PrettyPrinter/Delaborator/Builtins.lean b/src/Lean/PrettyPrinter/Delaborator/Builtins.lean index 68051e96ea3a..aa13f8f2c5cb 100644 --- a/src/Lean/PrettyPrinter/Delaborator/Builtins.lean +++ b/src/Lean/PrettyPrinter/Delaborator/Builtins.lean @@ -1014,7 +1014,7 @@ Delaborates an `OfNat.ofNat` literal. `@OfNat.ofNat _ n _` ~> `n`. -/ @[builtin_delab app.OfNat.ofNat] -def delabOfNat : Delab := whenPPOption getPPCoercions <| withOverApp 3 do +def delabOfNat : Delab := whenNotPPOption getPPExplicit <| whenPPOption getPPCoercions <| withOverApp 3 do delabOfNatCore (showType := (← getPPOption getPPNumericTypes)) /-- @@ -1022,7 +1022,7 @@ Delaborates the negative of an `OfNat.ofNat` literal. `-@OfNat.ofNat _ n _` ~> `-n` -/ @[builtin_delab app.Neg.neg] -def delabNeg : Delab := whenPPOption getPPCoercions do +def delabNeg : Delab := whenNotPPOption getPPExplicit <| whenPPOption getPPCoercions do delabNegIntCore (showType := (← getPPOption getPPNumericTypes)) /-- @@ -1031,12 +1031,12 @@ Delaborates a rational number literal. and `-@OfNat.ofNat _ n _ / @OfNat.ofNat _ m` ~> `-n / m` -/ @[builtin_delab app.HDiv.hDiv] -def delabHDiv : Delab := whenPPOption getPPCoercions do +def delabHDiv : Delab := whenNotPPOption getPPExplicit <| whenPPOption getPPCoercions do delabDivRatCore (showType := (← getPPOption getPPNumericTypes)) -- `@OfDecimal.ofDecimal _ _ m s e` ~> `m*10^(sign * e)` where `sign == 1` if `s = false` and `sign = -1` if `s = true` @[builtin_delab app.OfScientific.ofScientific] -def delabOfScientific : Delab := whenPPOption getPPCoercions <| withOverApp 5 do +def delabOfScientific : Delab := whenNotPPOption getPPExplicit <| whenPPOption getPPCoercions <| withOverApp 5 do let expr ← getExpr guard <| expr.getAppNumArgs == 5 let .lit (.natVal m) ← pure (expr.getArg! 2) | failure @@ -1080,6 +1080,9 @@ def coeDelaborator : Delab := whenPPOption getPPCoercions do let e ← getExpr let .const declName _ := e.getAppFn | failure let some info ← Meta.getCoeFnInfo? declName | failure + if (← getPPOption getPPExplicit) && info.coercee != 0 then + -- Approximation: the only implicit arguments come before the coercee + failure let n := e.getAppNumArgs withOverApp info.numArgs do match info.type with @@ -1092,7 +1095,7 @@ def coeDelaborator : Delab := whenPPOption getPPCoercions do | .coeSort => `(↥$(← withNaryArg info.coercee delab)) @[builtin_delab app.dite] -def delabDIte : Delab := whenPPOption getPPNotation <| withOverApp 5 do +def delabDIte : Delab := whenNotPPOption getPPExplicit <| whenPPOption getPPNotation <| withOverApp 5 do -- Note: we keep this as a delaborator for now because it actually accesses the expression. guard $ (← getExpr).getAppNumArgs == 5 let c ← withAppFn $ withAppFn $ withAppFn $ withAppArg delab @@ -1109,7 +1112,7 @@ where return (← delab, h.getId) @[builtin_delab app.cond] -def delabCond : Delab := whenPPOption getPPNotation <| withOverApp 4 do +def delabCond : Delab := whenNotPPOption getPPExplicit <| whenPPOption getPPNotation <| withOverApp 4 do guard $ (← getExpr).getAppNumArgs == 4 let c ← withAppFn $ withAppFn $ withAppArg delab let t ← withAppFn $ withAppArg delab @@ -1129,7 +1132,7 @@ def delabNamedPattern : Delab := do `($x:ident@$h:ident:$p:term) -- Sigma and PSigma delaborators -def delabSigmaCore (sigma : Bool) : Delab := whenPPOption getPPNotation do +def delabSigmaCore (sigma : Bool) : Delab := whenNotPPOption getPPExplicit <| whenPPOption getPPNotation do guard $ (← getExpr).getAppNumArgs == 2 guard $ (← getExpr).appArg!.isLambda withAppArg do @@ -1209,7 +1212,7 @@ partial def delabDoElems : DelabM (List Syntax) := do prependAndRec x : DelabM _ := List.cons <$> x <*> delabDoElems @[builtin_delab app.Bind.bind] -def delabDo : Delab := whenPPOption getPPNotation do +def delabDo : Delab := whenNotPPOption getPPExplicit <| whenPPOption getPPNotation do guard <| (← getExpr).isAppOfArity ``Bind.bind 6 let elems ← delabDoElems let items ← elems.toArray.mapM (`(doSeqItem|$(·):doElem)) diff --git a/src/Lean/Server/Completion.lean b/src/Lean/Server/Completion.lean index bb0829f4b0e2..83a38dac54aa 100644 --- a/src/Lean/Server/Completion.lean +++ b/src/Lean/Server/Completion.lean @@ -207,6 +207,8 @@ private def getCompletionKindForDecl (constInfo : ConstantInfo) : M CompletionIt return CompletionItemKind.enum else return CompletionItemKind.struct + else if constInfo.isTheorem then + return CompletionItemKind.event else if (← isProjectionFn constInfo.name) then return CompletionItemKind.field else if (← whnf constInfo.type).isForall then diff --git a/src/Lean/Structure.lean b/src/Lean/Structure.lean index 2d20b3280bea..519874b90e6c 100644 --- a/src/Lean/Structure.lean +++ b/src/Lean/Structure.lean @@ -8,25 +8,61 @@ Helper functions for retrieving structure information. prelude import Lean.Environment import Lean.ProjFns +import Lean.Exception namespace Lean +/-- +Data for a structure field. +These are direct fields of a structure, including "subobject" fields for the embedded parents. +The full collection of fields is the transitive closure of fields through the subobject fields. +-/ structure StructureFieldInfo where + /-- The name of the field. This is a single-component name. -/ fieldName : Name + /-- The projection function associated to the field. -/ projFn : Name - /-- It is `some parentStructName` if it is a subobject, and `parentStructName` is the name of the parent structure -/ + /-- If this field is for a subobject (i.e., an embedded parent structure), contains the name of the parent structure. -/ subobject? : Option Name + /-- The binder info for the field from the `structure` definition. -/ binderInfo : BinderInfo + /-- If set, the field is an autoparam (a field declared using `fld := by ...` syntax). + The expression evaluates to a tactic `Syntax` object. Generally this is an `Expr.const` expression. -/ autoParam? : Option Expr := none deriving Inhabited, Repr def StructureFieldInfo.lt (i₁ i₂ : StructureFieldInfo) : Bool := Name.quickLt i₁.fieldName i₂.fieldName -structure StructureInfo where +/-- +Data for a direct parent of a structure. +Some structure parents are represented as subobjects (embedded structures), +and for these the parent projection is a true projection. +If a structure parent shares a field with a previous parent, it will become an implicit parent, +and all the fields of the structure parent that do not occur in earlier parents are fields of the new structure +-/ +structure StructureParentInfo where + /-- The name of the parent structure. -/ structName : Name - fieldNames : Array Name := #[] -- sorted by field position in the structure - fieldInfo : Array StructureFieldInfo := #[] -- sorted by `fieldName` + /-- Whether this parent structure is represented as a subobject. If so, then there is a `fieldInfo` entry with the same `projFn`. -/ + subobject : Bool + /-- The projection function associated to the field. For subobjects, this is the same as the `projFn` in its `fieldInfo` entry. -/ + projFn : Name + deriving Inhabited + +/-- +Data about a type created with the `structure` command. +-/ +structure StructureInfo where + /-- The name of the structure. -/ + structName : Name + /-- The direct fields of a structure, sorted by position in the structure. + For example, the `s.3` notation refers to `fieldNames[3 - 1]`. -/ + fieldNames : Array Name := #[] + /-- Information about the structure fields, sorted by `fieldName`. -/ + fieldInfo : Array StructureFieldInfo := #[] + /-- (Unimplemented) Information about structure parents. These are in the order they appear in the `extends` clause. -/ + private parentInfo : Array StructureParentInfo := #[] deriving Inhabited def StructureInfo.lt (i₁ i₂ : StructureInfo) : Bool := @@ -50,11 +86,21 @@ builtin_initialize structureExt : SimplePersistentEnvExtension StructureInfo Str toArrayFn := fun es => es.toArray.qsort StructureInfo.lt } +/-- +A descriptor for a structure, for constructing a `StructureInfo` via `Lean.registerStructure`. +-/ structure StructureDescr where - structName : Name - fields : Array StructureFieldInfo -- Should use the order the field appear in the constructor. + /-- The name of the structure. -/ + structName : Name + /-- The fields should be in the order that they appear in the structure's constructor. -/ + fields : Array StructureFieldInfo deriving Inhabited +/-- +Declare a new structure to the elaborator. +Every structure created by `structure` or `class` has such an entry. +This should be followed up with `setStructureParents` and `setStructureResolutionOrder`. +-/ def registerStructure (env : Environment) (e : StructureDescr) : Environment := structureExt.addEntry env { structName := e.structName @@ -62,6 +108,15 @@ def registerStructure (env : Environment) (e : StructureDescr) : Environment := fieldInfo := e.fields.qsort StructureFieldInfo.lt } +/-- +Set parent projection info for a structure defined in the current module. +Throws an error if the structure has not already been registered with `Lean.registerStructure`. +-/ +def setStructureParents [Monad m] [MonadEnv m] [MonadError m] (structName : Name) (parentInfo : Array StructureParentInfo) : m Unit := do + let some info := structureExt.getState (← getEnv) |>.map.find? structName + | throwError "cannot set structure parents for '{structName}', structure not defined in current module" + modifyEnv fun env => structureExt.addEntry env { info with parentInfo } + def getStructureInfo? (env : Environment) (structName : Name) : Option StructureInfo := match env.getModuleIdxFor? structName with | some modIdx => structureExt.getModuleEntries env modIdx |>.binSearch { structName } StructureInfo.lt diff --git a/src/Lean/SubExpr.lean b/src/Lean/SubExpr.lean index 567b7da20dca..309eda5857c3 100644 --- a/src/Lean/SubExpr.lean +++ b/src/Lean/SubExpr.lean @@ -7,6 +7,7 @@ prelude import Lean.Meta.Basic import Lean.Data.Json import Lean.Data.RBMap +import Init.Control.Option namespace Lean diff --git a/src/Std/Tactic/BVDecide/Bitblast/BVExpr/Basic.lean b/src/Std/Tactic/BVDecide/Bitblast/BVExpr/Basic.lean index 48637e6eb2bd..d809340d14b7 100644 --- a/src/Std/Tactic/BVDecide/Bitblast/BVExpr/Basic.lean +++ b/src/Std/Tactic/BVDecide/Bitblast/BVExpr/Basic.lean @@ -73,6 +73,10 @@ inductive BVBinOp where Unsigned modulo. -/ | umod + /-- + Signed division. + -/ + | sdiv namespace BVBinOp @@ -84,6 +88,7 @@ def toString : BVBinOp → String | mul => "*" | udiv => "/ᵤ" | umod => "%ᵤ" + | sdiv => "/ₛ" instance : ToString BVBinOp := ⟨toString⟩ @@ -98,6 +103,7 @@ def eval : BVBinOp → (BitVec w → BitVec w → BitVec w) | mul => (· * ·) | udiv => (· / ·) | umod => (· % · ) + | sdiv => BitVec.sdiv @[simp] theorem eval_and : eval .and = ((· &&& ·) : BitVec w → BitVec w → BitVec w) := by rfl @[simp] theorem eval_or : eval .or = ((· ||| ·) : BitVec w → BitVec w → BitVec w) := by rfl @@ -106,6 +112,7 @@ def eval : BVBinOp → (BitVec w → BitVec w → BitVec w) @[simp] theorem eval_mul : eval .mul = ((· * ·) : BitVec w → BitVec w → BitVec w) := by rfl @[simp] theorem eval_udiv : eval .udiv = ((· / ·) : BitVec w → BitVec w → BitVec w) := by rfl @[simp] theorem eval_umod : eval .umod = ((· % ·) : BitVec w → BitVec w → BitVec w) := by rfl +@[simp] theorem eval_sdiv : eval .sdiv = (BitVec.sdiv : BitVec w → BitVec w → BitVec w) := by rfl end BVBinOp diff --git a/src/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Impl/Expr.lean b/src/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Impl/Expr.lean index 4e9e5bd87eca..ea9095ff18fe 100644 --- a/src/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Impl/Expr.lean +++ b/src/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Impl/Expr.lean @@ -21,6 +21,7 @@ import Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.SignExtend import Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Mul import Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Udiv import Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Umod +import Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Sdiv /-! This module contains the implementation of a bitblaster for `BitVec` expressions (`BVExpr`). @@ -117,6 +118,13 @@ where dsimp only at hlaig hraig omega ⟨res, this⟩ + | .sdiv => + let res := bitblast.blastSdiv aig ⟨lhs, rhs⟩ + have := by + apply AIG.LawfulVecOperator.le_size_of_le_aig_size (f := bitblast.blastSdiv) + dsimp only at hlaig hraig + omega + ⟨res, this⟩ | .un op expr => let ⟨⟨eaig, evec⟩, heaig⟩ := go aig expr match op with @@ -227,7 +235,7 @@ theorem bitblast.go_decl_eq (aig : AIG BVBit) (expr : BVExpr w) : rw [AIG.LawfulVecOperator.decl_eq (f := blastConst)] | bin lhs op rhs lih rih => match op with - | .and | .or | .xor | .add | .mul | .udiv | .umod => + | .and | .or | .xor | .add | .mul | .udiv | .umod | .sdiv => dsimp only [go] have := (bitblast.go aig lhs).property have := (go (go aig lhs).1.aig rhs).property diff --git a/src/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Impl/Operations/Sdiv.lean b/src/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Impl/Operations/Sdiv.lean new file mode 100644 index 000000000000..996cc28232d8 --- /dev/null +++ b/src/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Impl/Operations/Sdiv.lean @@ -0,0 +1,230 @@ +/- +Copyright (c) 2024 Lean FRO, LLC. All rights reserved. +Released under Apache 2.0 license as described in the file LICENSE. +Authors: Henrik Böving +-/ +prelude +import Std.Sat.AIG.If +import Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Neg +import Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Udiv + +/-! +This module contains the implementation of a bitblaster for `BitVec.sdiv`. The implemented +circuit is the reduction to udiv. +-/ + +namespace Std.Tactic.BVDecide + +open Std.Sat + +namespace BVExpr +namespace bitblast + +variable [Hashable α] [DecidableEq α] + +namespace blastSdiv + +structure SignBranchInput (aig : AIG α) (len : Nat) where + w : Nat + lhs : AIG.RefVec aig w + rhs : AIG.RefVec aig w + lposRpos : AIG.RefVec aig len + lposRneg : AIG.RefVec aig len + lnegRpos : AIG.RefVec aig len + lnegRneg : AIG.RefVec aig len + hnezero : w ≠ 0 + +def signBranch (aig : AIG α) (input : SignBranchInput aig len) : AIG.RefVecEntry α len := + let ⟨w, lhs, rhs, lposRpos, lposRneg, lnegRpos, lnegRneg, hnezero⟩ := input + let res := AIG.RefVec.ite aig ⟨rhs.get (w - 1) (by omega), lposRneg, lposRpos⟩ + let aig := res.aig + let lposHalf := res.vec + have := AIG.LawfulVecOperator.le_size (f := AIG.RefVec.ite) .. + let lhs := lhs.cast this + let rhs := rhs.cast this + let lnegRneg := lnegRneg.cast this + let lnegRpos := lnegRpos.cast this + + let res := AIG.RefVec.ite aig ⟨rhs.get (w - 1) (by omega), lnegRneg, lnegRpos⟩ + let aig := res.aig + let lnegHalf := res.vec + have := AIG.LawfulVecOperator.le_size (f := AIG.RefVec.ite) .. + let lhs := lhs.cast this + let lposHalf := lposHalf.cast this + + AIG.RefVec.ite aig ⟨lhs.get (w - 1) (by omega), lnegHalf, lposHalf⟩ + +instance : AIG.LawfulVecOperator α SignBranchInput signBranch where + le_size := by + intros + unfold signBranch + dsimp only + apply AIG.LawfulVecOperator.le_size_of_le_aig_size (f := AIG.RefVec.ite) + apply AIG.LawfulVecOperator.le_size_of_le_aig_size (f := AIG.RefVec.ite) + apply AIG.LawfulVecOperator.le_size (f := AIG.RefVec.ite) + decl_eq := by + intros + unfold signBranch + dsimp only + rw [AIG.LawfulVecOperator.decl_eq (f := AIG.RefVec.ite)] + rw [AIG.LawfulVecOperator.decl_eq (f := AIG.RefVec.ite)] + rw [AIG.LawfulVecOperator.decl_eq (f := AIG.RefVec.ite)] + · apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := AIG.RefVec.ite) + assumption + · apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := AIG.RefVec.ite) + apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := AIG.RefVec.ite) + assumption + +end blastSdiv + +def blastSdiv (aig : AIG α) (input : AIG.BinaryRefVec aig w) : AIG.RefVecEntry α w := + if h : w = 0 then + ⟨aig, h ▸ AIG.RefVec.empty⟩ + else + let ⟨lhs, rhs⟩ := input + let res := blastNeg aig lhs + let aig := res.aig + let negLhs := res.vec + have := AIG.LawfulVecOperator.le_size (f := blastNeg) .. + let lhs := lhs.cast this + let rhs := rhs.cast this + let res := blastNeg aig rhs + let aig := res.aig + let negRhs := res.vec + have := AIG.LawfulVecOperator.le_size (f := blastNeg) .. + let lhs := lhs.cast this + let rhs := rhs.cast this + let negLhs := negLhs.cast this + + let res := blastUdiv aig ⟨lhs, rhs⟩ + let aig := res.aig + let lposRpos := res.vec + have := AIG.LawfulVecOperator.le_size (f := blastUdiv) .. + let lhs := lhs.cast this + let rhs := rhs.cast this + let negRhs := negRhs.cast this + let negLhs := negLhs.cast this + + let res := blastUdiv aig ⟨lhs, negRhs⟩ + let aig := res.aig + let ldivnr := res.vec + let res := blastNeg aig ldivnr + let aig := res.aig + let lposRneg := res.vec + have := by + apply AIG.LawfulVecOperator.le_size_of_le_aig_size (f := blastNeg) + apply AIG.LawfulVecOperator.le_size (f := blastUdiv) + let lhs := lhs.cast this + let rhs := rhs.cast this + let negRhs := negRhs.cast this + let negLhs := negLhs.cast this + let lposRpos := lposRpos.cast this + + let res := blastUdiv aig ⟨negLhs, rhs⟩ + let aig := res.aig + let nldivr := res.vec + let res := blastNeg aig nldivr + let aig := res.aig + let lnegRpos := res.vec + have := by + apply AIG.LawfulVecOperator.le_size_of_le_aig_size (f := blastNeg) + apply AIG.LawfulVecOperator.le_size (f := blastUdiv) + let lhs := lhs.cast this + let rhs := rhs.cast this + let negRhs := negRhs.cast this + let negLhs := negLhs.cast this + let lposRpos := lposRpos.cast this + let lposRneg := lposRneg.cast this + + let res := blastUdiv aig ⟨negLhs, negRhs⟩ + let aig := res.aig + let lnegRneg := res.vec + have := AIG.LawfulVecOperator.le_size (f := blastUdiv) .. + let lhs := lhs.cast this + let rhs := rhs.cast this + let lposRpos := lposRpos.cast this + let lposRneg := lposRneg.cast this + let lnegRpos := lnegRpos.cast this + + blastSdiv.signBranch aig ⟨w, lhs, rhs, lposRpos, lposRneg, lnegRpos, lnegRneg, h⟩ + +instance : AIG.LawfulVecOperator α AIG.BinaryRefVec blastSdiv where + le_size := by + intros + unfold blastSdiv + dsimp only + split + · simp + · apply AIG.LawfulVecOperator.le_size_of_le_aig_size (f := blastSdiv.signBranch) + apply AIG.LawfulVecOperator.le_size_of_le_aig_size (f := blastUdiv) + apply AIG.LawfulVecOperator.le_size_of_le_aig_size (f := blastNeg) + apply AIG.LawfulVecOperator.le_size_of_le_aig_size (f := blastUdiv) + apply AIG.LawfulVecOperator.le_size_of_le_aig_size (f := blastNeg) + apply AIG.LawfulVecOperator.le_size_of_le_aig_size (f := blastUdiv) + apply AIG.LawfulVecOperator.le_size_of_le_aig_size (f := blastUdiv) + apply AIG.LawfulVecOperator.le_size_of_le_aig_size (f := blastNeg) + apply AIG.LawfulVecOperator.le_size (f := blastNeg) + decl_eq := by + intros + unfold blastSdiv + dsimp only + split + · simp + · rw [AIG.LawfulVecOperator.decl_eq (f := blastSdiv.signBranch)] + rw [AIG.LawfulVecOperator.decl_eq (f := blastUdiv)] + rw [AIG.LawfulVecOperator.decl_eq (f := blastNeg)] + rw [AIG.LawfulVecOperator.decl_eq (f := blastUdiv)] + rw [AIG.LawfulVecOperator.decl_eq (f := blastNeg)] + rw [AIG.LawfulVecOperator.decl_eq (f := blastUdiv)] + rw [AIG.LawfulVecOperator.decl_eq (f := blastUdiv)] + rw [AIG.LawfulVecOperator.decl_eq (f := blastNeg)] + rw [AIG.LawfulVecOperator.decl_eq (f := blastNeg)] + · apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastNeg) + assumption + · apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastNeg) + apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastNeg) + assumption + · apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastUdiv) + apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastNeg) + apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastNeg) + assumption + · apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastUdiv) + apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastUdiv) + apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastNeg) + apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastNeg) + assumption + · apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastNeg) + apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastUdiv) + apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastUdiv) + apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastNeg) + apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastNeg) + assumption + · apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastUdiv) + apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastNeg) + apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastUdiv) + apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastUdiv) + apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastNeg) + apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastNeg) + assumption + · apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastNeg) + apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastUdiv) + apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastNeg) + apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastUdiv) + apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastUdiv) + apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastNeg) + apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastNeg) + assumption + · apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastUdiv) + apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastNeg) + apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastUdiv) + apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastNeg) + apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastUdiv) + apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastUdiv) + apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastNeg) + apply AIG.LawfulVecOperator.lt_size_of_lt_aig_size (f := blastNeg) + assumption + +end bitblast +end BVExpr + +end Std.Tactic.BVDecide diff --git a/src/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Lemmas/Expr.lean b/src/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Lemmas/Expr.lean index 6c7d5e29f6d4..1475225804ca 100644 --- a/src/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Lemmas/Expr.lean +++ b/src/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Lemmas/Expr.lean @@ -21,6 +21,7 @@ import Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.SignExtend import Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.Mul import Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.Udiv import Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.Umod +import Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.Sdiv import Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Expr /-! @@ -218,6 +219,18 @@ theorem go_denote_eq (aig : AIG BVBit) (expr : BVExpr w) (assign : Assignment) : · simp [Ref.hgate] · intros rw [← rih] + | sdiv => + simp only [go, eval_bin, BVBinOp.eval_sdiv] + apply denote_blastSdiv + · intros + dsimp only + rw [go_denote_mem_prefix] + rw [← lih (aig := aig)] + · simp + · assumption + · simp [Ref.hgate] + · intros + rw [← rih] | un op expr ih => cases op with | not => simp [go, ih, hidx] diff --git a/src/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Lemmas/Operations/Sdiv.lean b/src/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Lemmas/Operations/Sdiv.lean new file mode 100644 index 000000000000..9ba6ed8abe5c --- /dev/null +++ b/src/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Lemmas/Operations/Sdiv.lean @@ -0,0 +1,201 @@ +/- +Copyright (c) 2024 Lean FRO, LLC. All rights reserved. +Released under Apache 2.0 license as described in the file LICENSE. +Authors: Henrik Böving +-/ +prelude +import Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.Udiv +import Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.Neg +import Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Sdiv +import Std.Tactic.BVDecide.Normalize.BitVec + +/-! +This module contains the verification of the `BitVec.sdiv` bitblaster from `Impl.Operations.Sdiv`. +-/ + +namespace Std.Tactic.BVDecide + +open Std.Sat +open Std.Sat.AIG + +namespace BVExpr +namespace bitblast + +variable [Hashable α] [DecidableEq α] + +namespace blastSdiv + +theorem denote_signBranch {aig : AIG α} (input : SignBranchInput aig len) (lhs rhs : BitVec input.w) + (lposRpos lposRneg lnegRpos lnegRneg : BitVec len) + (hleft : ∀ (idx : Nat) (hidx : idx < input.w), ⟦aig, input.lhs.get idx hidx, assign⟧ = lhs.getLsbD idx) + (hright : ∀ (idx : Nat) (hidx : idx < input.w), ⟦aig, input.rhs.get idx hidx, assign⟧ = rhs.getLsbD idx) + (hlprp : ∀ (idx : Nat) (hidx : idx < len), ⟦aig, input.lposRpos.get idx hidx, assign⟧ = lposRpos.getLsbD idx) + (hlprn : ∀ (idx : Nat) (hidx : idx < len), ⟦aig, input.lposRneg.get idx hidx, assign⟧ = lposRneg.getLsbD idx) + (hlnrp : ∀ (idx : Nat) (hidx : idx < len), ⟦aig, input.lnegRpos.get idx hidx, assign⟧ = lnegRpos.getLsbD idx) + (hlnrn : ∀ (idx : Nat) (hidx : idx < len), ⟦aig, input.lnegRneg.get idx hidx, assign⟧ = lnegRneg.getLsbD idx) : + ∀ (idx : Nat) (hidx : idx < len), + ⟦(signBranch aig input).aig, (signBranch aig input).vec.get idx hidx, assign⟧ + = + (match lhs.msb, rhs.msb with + | false, false => lposRpos + | false, true => lposRneg + | true, false => lnegRpos + | true, true => lnegRneg).getLsbD idx + := by + intros + unfold signBranch + simp only [ne_eq, RefVec.denote_ite, RefVec.get_cast, Ref.cast_eq] + split + · next h1 => + rw [AIG.LawfulVecOperator.denote_mem_prefix, AIG.LawfulVecOperator.denote_mem_prefix] at h1 + rw [hleft, ← BitVec.msb_eq_getLsbD_last] at h1 + rw [h1] + split + · next h2 => + rw [AIG.LawfulVecOperator.denote_mem_prefix] at h2 + rw [hright, ← BitVec.msb_eq_getLsbD_last] at h2 + rw [h2] + rw [AIG.LawfulVecOperator.denote_mem_prefix, hlnrn] + · next h2 => + rw [AIG.LawfulVecOperator.denote_mem_prefix] at h2 + rw [hright, ← BitVec.msb_eq_getLsbD_last, Bool.not_eq_true] at h2 + rw [h2] + rw [AIG.LawfulVecOperator.denote_mem_prefix, hlnrp] + · next h1 => + rw [AIG.LawfulVecOperator.denote_mem_prefix, AIG.LawfulVecOperator.denote_mem_prefix] at h1 + rw [hleft, ← BitVec.msb_eq_getLsbD_last, Bool.not_eq_true] at h1 + rw [h1] + rw [AIG.LawfulVecOperator.denote_mem_prefix] + rw [AIG.RefVec.denote_ite] + split + · next h2 => + rw [hright, ← BitVec.msb_eq_getLsbD_last] at h2 + rw [h2] + simp [hlprn] + · next h2 => + rw [hright, ← BitVec.msb_eq_getLsbD_last, Bool.not_eq_true] at h2 + rw [h2] + simp [hlprp] + +end blastSdiv + +theorem denote_blastSdiv (aig : AIG α) (lhs rhs : BitVec w) (assign : α → Bool) + (input : BinaryRefVec aig w) + (hleft : ∀ (idx : Nat) (hidx : idx < w), ⟦aig, input.lhs.get idx hidx, assign⟧ = lhs.getLsbD idx) + (hright : ∀ (idx : Nat) (hidx : idx < w), ⟦aig, input.rhs.get idx hidx, assign⟧ = rhs.getLsbD idx) : + ∀ (idx : Nat) (hidx : idx < w), + ⟦(blastSdiv aig input).aig, (blastSdiv aig input).vec.get idx hidx, assign⟧ + = + (BitVec.sdiv lhs rhs).getLsbD idx := by + intros + generalize hres : blastSdiv aig input = res + unfold blastSdiv at hres + split at hres + · omega + · dsimp only at hres + rw [← hres] + clear hres + rw [blastSdiv.denote_signBranch + (lhs := lhs) + (rhs := rhs) + (lposRpos := lhs / rhs) + (lposRneg := -(lhs / (-rhs))) + (lnegRpos := -((-lhs) / rhs)) + (lnegRneg := ((-lhs) / (-rhs))) + ] + · rw [BitVec.sdiv_eq] + rfl + · simp only [RefVec.get_cast, Ref.cast_eq] + intros + rw [AIG.LawfulVecOperator.denote_mem_prefix, AIG.LawfulVecOperator.denote_mem_prefix, + AIG.LawfulVecOperator.denote_mem_prefix, AIG.LawfulVecOperator.denote_mem_prefix, + AIG.LawfulVecOperator.denote_mem_prefix, AIG.LawfulVecOperator.denote_mem_prefix, + AIG.LawfulVecOperator.denote_mem_prefix, AIG.LawfulVecOperator.denote_mem_prefix] + rw [hleft] + · simp only [RefVec.get_cast, Ref.cast_eq] + intros + rw [AIG.LawfulVecOperator.denote_mem_prefix, AIG.LawfulVecOperator.denote_mem_prefix, + AIG.LawfulVecOperator.denote_mem_prefix, AIG.LawfulVecOperator.denote_mem_prefix, + AIG.LawfulVecOperator.denote_mem_prefix, AIG.LawfulVecOperator.denote_mem_prefix, + AIG.LawfulVecOperator.denote_mem_prefix, AIG.LawfulVecOperator.denote_mem_prefix] + rw [hright] + · simp only [RefVec.get_cast, Ref.cast_eq] + intros + rw [AIG.LawfulVecOperator.denote_mem_prefix, AIG.LawfulVecOperator.denote_mem_prefix, + AIG.LawfulVecOperator.denote_mem_prefix, AIG.LawfulVecOperator.denote_mem_prefix, + AIG.LawfulVecOperator.denote_mem_prefix] + rw [denote_blastUdiv (lhs := lhs) (rhs := rhs)] + · intros + rw [AIG.LawfulVecOperator.denote_mem_prefix, AIG.LawfulVecOperator.denote_mem_prefix] + · simp [hleft] + · simp [Ref.hgate] + · intros + rw [AIG.LawfulVecOperator.denote_mem_prefix, AIG.LawfulVecOperator.denote_mem_prefix] + · simp [hright] + · simp [Ref.hgate] + · simp only [RefVec.get_cast, Ref.cast_eq] + intros + rw [AIG.LawfulVecOperator.denote_mem_prefix, AIG.LawfulVecOperator.denote_mem_prefix, + AIG.LawfulVecOperator.denote_mem_prefix] + rw [denote_blastNeg (value := lhs / (-rhs))] + intros + rw [denote_blastUdiv (lhs := lhs) (rhs := -rhs)] + · intros + rw [AIG.LawfulVecOperator.denote_mem_prefix, AIG.LawfulVecOperator.denote_mem_prefix, + AIG.LawfulVecOperator.denote_mem_prefix] + · simp [hleft] + · simp [Ref.hgate] + · intros + rw [AIG.LawfulVecOperator.denote_mem_prefix] + · simp only [RefVec.get_cast, Ref.cast_eq] + rw [denote_blastNeg (value := rhs)] + intros + rw [AIG.LawfulVecOperator.denote_mem_prefix] + · simp [hright] + · simp [Ref.hgate] + · simp [Ref.hgate] + · simp only [RefVec.get_cast, Ref.cast_eq] + intros + rw [AIG.LawfulVecOperator.denote_mem_prefix] + rw [denote_blastNeg (value := (-lhs) / rhs)] + intros + rw [denote_blastUdiv (lhs := -lhs) (rhs := rhs)] + · intros + rw [AIG.LawfulVecOperator.denote_mem_prefix, AIG.LawfulVecOperator.denote_mem_prefix, + AIG.LawfulVecOperator.denote_mem_prefix, AIG.LawfulVecOperator.denote_mem_prefix] + · simp only [RefVec.get_cast, Ref.cast_eq] + rw [denote_blastNeg (value := lhs)] + simp [hleft] + · simp [Ref.hgate] + · intros + rw [AIG.LawfulVecOperator.denote_mem_prefix, AIG.LawfulVecOperator.denote_mem_prefix, + AIG.LawfulVecOperator.denote_mem_prefix, AIG.LawfulVecOperator.denote_mem_prefix, + AIG.LawfulVecOperator.denote_mem_prefix] + · simp [hright] + · simp [Ref.hgate] + · simp only + intros + rw [denote_blastUdiv (lhs := -lhs) (rhs := - rhs)] + · intros + simp only [RefVec.get_cast, Ref.cast_eq] + rw [AIG.LawfulVecOperator.denote_mem_prefix, AIG.LawfulVecOperator.denote_mem_prefix, + AIG.LawfulVecOperator.denote_mem_prefix, AIG.LawfulVecOperator.denote_mem_prefix, + AIG.LawfulVecOperator.denote_mem_prefix, AIG.LawfulVecOperator.denote_mem_prefix] + rw [denote_blastNeg (value := lhs)] + simp [hleft] + · intros + simp only [RefVec.get_cast, Ref.cast_eq] + rw [AIG.LawfulVecOperator.denote_mem_prefix, AIG.LawfulVecOperator.denote_mem_prefix, + AIG.LawfulVecOperator.denote_mem_prefix, AIG.LawfulVecOperator.denote_mem_prefix, + AIG.LawfulVecOperator.denote_mem_prefix] + rw [denote_blastNeg (value := rhs)] + intros + rw [AIG.LawfulVecOperator.denote_mem_prefix] + · simp [hright] + · simp [Ref.hgate] + + +end bitblast +end BVExpr + +end Std.Tactic.BVDecide diff --git a/src/Std/Tactic/BVDecide/Normalize/BitVec.lean b/src/Std/Tactic/BVDecide/Normalize/BitVec.lean index f2a4d4ad61ae..95c2a7ce3c44 100644 --- a/src/Std/Tactic/BVDecide/Normalize/BitVec.lean +++ b/src/Std/Tactic/BVDecide/Normalize/BitVec.lean @@ -262,6 +262,7 @@ attribute [bv_normalize] BitVec.zero_umod attribute [bv_normalize] BitVec.umod_zero attribute [bv_normalize] BitVec.umod_one attribute [bv_normalize] BitVec.umod_eq_and +attribute [bv_normalize] BitVec.sdiv_eq_and end Normalize end Std.Tactic.BVDecide diff --git a/src/Std/Tactic/BVDecide/Reflect.lean b/src/Std/Tactic/BVDecide/Reflect.lean index aebaba3b7b00..93e729b537ed 100644 --- a/src/Std/Tactic/BVDecide/Reflect.lean +++ b/src/Std/Tactic/BVDecide/Reflect.lean @@ -118,6 +118,10 @@ theorem umod_congr (lhs rhs lhs' rhs' : BitVec w) (h1 : lhs' = lhs) (h2 : rhs' = (lhs' % rhs') = (lhs % rhs) := by simp[*] +theorem sdiv_congr (lhs rhs lhs' rhs' : BitVec w) (h1 : lhs' = lhs) (h2 : rhs' = rhs) : + (BitVec.sdiv lhs' rhs') = (BitVec.sdiv lhs rhs) := by + simp[*] + end BitVec namespace Bool diff --git a/src/cmake/Modules/FindWindowsSDK.cmake b/src/cmake/Modules/FindWindowsSDK.cmake new file mode 100644 index 000000000000..17519ba59b18 --- /dev/null +++ b/src/cmake/Modules/FindWindowsSDK.cmake @@ -0,0 +1,643 @@ +# - Find the Windows SDK aka Platform SDK +# +# Relevant Wikipedia article: http://en.wikipedia.org/wiki/Microsoft_Windows_SDK +# +# Pass "COMPONENTS tools" to ignore Visual Studio version checks: in case +# you just want the tool binaries to run, rather than the libraries and headers +# for compiling. +# +# Variables: +# WINDOWSSDK_FOUND - if any version of the windows or platform SDK was found that is usable with the current version of visual studio +# WINDOWSSDK_LATEST_DIR +# WINDOWSSDK_LATEST_NAME +# WINDOWSSDK_FOUND_PREFERENCE - if we found an entry indicating a "preferred" SDK listed for this visual studio version +# WINDOWSSDK_PREFERRED_DIR +# WINDOWSSDK_PREFERRED_NAME +# +# WINDOWSSDK_DIRS - contains no duplicates, ordered most recent first. +# WINDOWSSDK_PREFERRED_FIRST_DIRS - contains no duplicates, ordered with preferred first, followed by the rest in descending recency +# +# Functions: +# windowssdk_name_lookup( ) - Find the name corresponding with the SDK directory you pass in, or +# NOTFOUND if not recognized. Your directory must be one of WINDOWSSDK_DIRS for this to work. +# +# windowssdk_build_lookup( ) - Find the build version number corresponding with the SDK directory you pass in, or +# NOTFOUND if not recognized. Your directory must be one of WINDOWSSDK_DIRS for this to work. +# +# get_windowssdk_from_component( ) - Given a library or include dir, +# find the Windows SDK root dir corresponding to it, or NOTFOUND if unrecognized. +# +# get_windowssdk_library_dirs( ) - Find the architecture-appropriate +# library directories corresponding to the SDK directory you pass in (or NOTFOUND if none) +# +# get_windowssdk_library_dirs_multiple( ...) - Find the architecture-appropriate +# library directories corresponding to the SDK directories you pass in, in order, skipping those not found. NOTFOUND if none at all. +# Good for passing WINDOWSSDK_DIRS or WINDOWSSDK_DIRS to if you really just want a file and don't care where from. +# +# get_windowssdk_include_dirs( ) - Find the +# include directories corresponding to the SDK directory you pass in (or NOTFOUND if none) +# +# get_windowssdk_include_dirs_multiple( ...) - Find the +# include directories corresponding to the SDK directories you pass in, in order, skipping those not found. NOTFOUND if none at all. +# Good for passing WINDOWSSDK_DIRS or WINDOWSSDK_DIRS to if you really just want a file and don't care where from. +# +# Requires these CMake modules: +# FindPackageHandleStandardArgs (known included with CMake >=2.6.2) +# +# Original Author: +# 2012 Rylie Pavlik +# https://ryliepavlik.com/ +# Iowa State University HCI Graduate Program/VRAC +# +# Copyright 2012, Iowa State University +# +# Distributed under the Boost Software License, Version 1.0. +# (See accompanying file LICENSE_1_0.txt or copy at +# http://www.boost.org/LICENSE_1_0.txt) +# +# SPDX-License-Identifier: BSL-1.0 + +set(_preferred_sdk_dirs) # pre-output +set(_win_sdk_dirs) # pre-output +set(_win_sdk_versanddirs) # pre-output +set(_win_sdk_buildsanddirs) # pre-output +set(_winsdk_vistaonly) # search parameters +set(_winsdk_kits) # search parameters + + +set(_WINDOWSSDK_ANNOUNCE OFF) +if(NOT WINDOWSSDK_FOUND AND (NOT WindowsSDK_FIND_QUIETLY)) + set(_WINDOWSSDK_ANNOUNCE ON) +endif() +macro(_winsdk_announce) + if(_WINSDK_ANNOUNCE) + message(STATUS ${ARGN}) + endif() +endmacro() + +# See https://developer.microsoft.com/en-us/windows/downloads/sdk-archive - +# although version numbers listed on that page don't necessarily match the directory +# used by the installer. +set(_winsdk_win10vers + 10.0.26100.0 + 10.0.22621.0 + 10.0.22000.0 + 10.0.20348.0 + 10.0.19041.0 + 10.0.18362.0 # Win10 1903 "19H1" + 10.0.17763.0 # Win10 1809 "October 2018 Update" + 10.0.17134.0 # Redstone 4 aka Win10 1803 "April 2018 Update" + 10.0.17133.0 # Redstone 4 aka Win10 1803 "April 2018 Update" + 10.0.16299.0 # Redstone 3 aka Win10 1709 "Fall Creators Update" + 10.0.15063.0 # Redstone 2 aka Win10 1703 "Creators Update" + 10.0.14393.0 # Redstone aka Win10 1607 "Anniversary Update" + 10.0.10586.0 # TH2 aka Win10 1511 + 10.0.10240.0 # Win10 RTM + 10.0.10150.0 # just ucrt + 10.0.10056.0 +) + +if(WindowsSDK_FIND_COMPONENTS MATCHES "tools") + set(_WINDOWSSDK_IGNOREMSVC ON) + _winsdk_announce("Checking for tools from Windows/Platform SDKs...") +else() + set(_WINDOWSSDK_IGNOREMSVC OFF) + _winsdk_announce("Checking for Windows/Platform SDKs...") +endif() + +# Appends to the three main pre-output lists used only if the path exists +# and is not already in the list. +function(_winsdk_conditional_append _vername _build _path) + if(("${_path}" MATCHES "registry") OR (NOT EXISTS "${_path}")) + # Path invalid - do not add + return() + endif() + list(FIND _win_sdk_dirs "${_path}" _win_sdk_idx) + if(_win_sdk_idx GREATER -1) + # Path already in list - do not add + return() + endif() + _winsdk_announce( " - ${_vername}, Build ${_build} @ ${_path}") + # Not yet in the list, so we'll add it + list(APPEND _win_sdk_dirs "${_path}") + set(_win_sdk_dirs "${_win_sdk_dirs}" CACHE INTERNAL "" FORCE) + list(APPEND + _win_sdk_versanddirs + "${_vername}" + "${_path}") + set(_win_sdk_versanddirs "${_win_sdk_versanddirs}" CACHE INTERNAL "" FORCE) + list(APPEND + _win_sdk_buildsanddirs + "${_build}" + "${_path}") + set(_win_sdk_buildsanddirs "${_win_sdk_buildsanddirs}" CACHE INTERNAL "" FORCE) +endfunction() + +# Appends to the "preferred SDK" lists only if the path exists +function(_winsdk_conditional_append_preferred _info _path) + if(("${_path}" MATCHES "registry") OR (NOT EXISTS "${_path}")) + # Path invalid - do not add + return() + endif() + + get_filename_component(_path "${_path}" ABSOLUTE) + + list(FIND _win_sdk_preferred_sdk_dirs "${_path}" _win_sdk_idx) + if(_win_sdk_idx GREATER -1) + # Path already in list - do not add + return() + endif() + _winsdk_announce( " - Found \"preferred\" SDK ${_info} @ ${_path}") + # Not yet in the list, so we'll add it + list(APPEND _win_sdk_preferred_sdk_dirs "${_path}") + set(_win_sdk_preferred_sdk_dirs "${_win_sdk_dirs}" CACHE INTERNAL "" FORCE) + + # Just in case we somehow missed it: + _winsdk_conditional_append("${_info}" "" "${_path}") +endfunction() + +# Given a version like v7.0A, looks for an SDK in the registry under "Microsoft SDKs". +# If the given version might be in both HKEY_LOCAL_MACHINE\\SOFTWARE\\Microsoft\\Microsoft SDKs\\Windows +# and HKEY_LOCAL_MACHINE\\SOFTWARE\\Microsoft\\Windows Kits\\Installed Roots aka "Windows Kits", +# use this macro first, since these registry keys usually have more information. +# +# Pass a "default" build number as an extra argument in case we can't find it. +function(_winsdk_check_microsoft_sdks_registry _winsdkver) + set(SDKKEY "HKEY_LOCAL_MACHINE\\SOFTWARE\\Microsoft\\Microsoft SDKs\\Windows\\${_winsdkver}") + get_filename_component(_sdkdir + "[${SDKKEY};InstallationFolder]" + ABSOLUTE) + + set(_sdkname "Windows SDK ${_winsdkver}") + + # Default build number passed as extra argument + set(_build ${ARGN}) + # See if the registry holds a Microsoft-mutilated, err, designated, product name + # (just using get_filename_component to execute the registry lookup) + get_filename_component(_sdkproductname + "[${SDKKEY};ProductName]" + NAME) + if(NOT "${_sdkproductname}" MATCHES "registry") + # Got a product name + set(_sdkname "${_sdkname} (${_sdkproductname})") + endif() + + # try for a version to augment our name + # (just using get_filename_component to execute the registry lookup) + get_filename_component(_sdkver + "[${SDKKEY};ProductVersion]" + NAME) + if(NOT "${_sdkver}" MATCHES "registry" AND NOT MATCHES) + # Got a version + if(NOT "${_sdkver}" MATCHES "\\.\\.") + # and it's not an invalid one with two dots in it: + # use to override the default build + set(_build ${_sdkver}) + if(NOT "${_sdkname}" MATCHES "${_sdkver}") + # Got a version that's not already in the name, let's use it to improve our name. + set(_sdkname "${_sdkname} (${_sdkver})") + endif() + endif() + endif() + _winsdk_conditional_append("${_sdkname}" "${_build}" "${_sdkdir}") +endfunction() + +# Given a name for identification purposes, the build number, and a key (technically a "value name") +# corresponding to a Windows SDK packaged as a "Windows Kit", look for it +# in HKEY_LOCAL_MACHINE\\SOFTWARE\\Microsoft\\Windows Kits\\Installed Roots +# Note that the key or "value name" tends to be something weird like KitsRoot81 - +# no easy way to predict, just have to observe them in the wild. +# Doesn't hurt to also try _winsdk_check_microsoft_sdks_registry for these: +# sometimes you get keys in both parts of the registry (in the wow64 portion especially), +# and the non-"Windows Kits" location is often more descriptive. +function(_winsdk_check_windows_kits_registry _winkit_name _winkit_build _winkit_key) + get_filename_component(_sdkdir + "[HKEY_LOCAL_MACHINE\\SOFTWARE\\Microsoft\\Windows Kits\\Installed Roots;${_winkit_key}]" + ABSOLUTE) + _winsdk_conditional_append("${_winkit_name}" "${_winkit_build}" "${_sdkdir}") +endfunction() + +# Given a name for identification purposes and the build number +# corresponding to a Windows 10 SDK packaged as a "Windows Kit", look for it +# in HKEY_LOCAL_MACHINE\\SOFTWARE\\Microsoft\\Windows Kits\\Installed Roots +# Doesn't hurt to also try _winsdk_check_microsoft_sdks_registry for these: +# sometimes you get keys in both parts of the registry (in the wow64 portion especially), +# and the non-"Windows Kits" location is often more descriptive. +function(_winsdk_check_win10_kits _winkit_build) + get_filename_component(_sdkdir + "[HKEY_LOCAL_MACHINE\\SOFTWARE\\Microsoft\\Windows Kits\\Installed Roots;KitsRoot10]" + ABSOLUTE) + if(("${_sdkdir}" MATCHES "registry") OR (NOT EXISTS "${_sdkdir}")) + return() # not found + endif() + if(EXISTS "${_sdkdir}/Include/${_winkit_build}/um") + _winsdk_conditional_append("Windows Kits 10 (Build ${_winkit_build})" "${_winkit_build}" "${_sdkdir}") + endif() +endfunction() + +# Given a name for indentification purposes, the build number, and the associated package GUID, +# look in the registry under both HKLM and HKCU in \\SOFTWARE\\Microsoft\\MicrosoftSDK\\InstalledSDKs\\ +# for that guid and the SDK it points to. +function(_winsdk_check_platformsdk_registry _platformsdkname _build _platformsdkguid) + foreach(_winsdk_hive HKEY_LOCAL_MACHINE HKEY_CURRENT_USER) + get_filename_component(_sdkdir + "[${_winsdk_hive}\\SOFTWARE\\Microsoft\\MicrosoftSDK\\InstalledSDKs\\${_platformsdkguid};Install Dir]" + ABSOLUTE) + _winsdk_conditional_append("${_platformsdkname} (${_build})" "${_build}" "${_sdkdir}") + endforeach() +endfunction() + +### +# Detect toolchain information: to know whether it's OK to use Vista+ only SDKs +### +set(_winsdk_vistaonly_ok OFF) +if(MSVC AND NOT _WINDOWSSDK_IGNOREMSVC) + # VC 10 and older has broad target support + if(MSVC_VERSION LESS 1700) + # VC 11 by default targets Vista and later only, so we can add a few more SDKs that (might?) only work on vista+ + elseif("${CMAKE_VS_PLATFORM_TOOLSET}" MATCHES "_xp") + # This is the XP-compatible v110+ toolset + elseif("${CMAKE_VS_PLATFORM_TOOLSET}" STREQUAL "v100" OR "${CMAKE_VS_PLATFORM_TOOLSET}" STREQUAL "v90") + # This is the VS2010/VS2008 toolset + else() + # OK, we're VC11 or newer and not using a backlevel or XP-compatible toolset. + # These versions have no XP (and possibly Vista pre-SP1) support + set(_winsdk_vistaonly_ok ON) + if(_WINDOWSSDK_ANNOUNCE AND NOT _WINDOWSSDK_VISTAONLY_PESTERED) + set(_WINDOWSSDK_VISTAONLY_PESTERED ON CACHE INTERNAL "" FORCE) + message(STATUS "FindWindowsSDK: Detected Visual Studio 2012 or newer, not using the _xp toolset variant: including SDK versions that drop XP support in search!") + endif() + endif() +endif() +if(_WINDOWSSDK_IGNOREMSVC) + set(_winsdk_vistaonly_ok ON) +endif() + +### +# MSVC version checks - keeps messy conditionals in one place +# (messy because of _WINDOWSSDK_IGNOREMSVC) +### +set(_winsdk_msvc_greater_1200 OFF) +if(_WINDOWSSDK_IGNOREMSVC OR (MSVC AND (MSVC_VERSION GREATER 1200))) + set(_winsdk_msvc_greater_1200 ON) +endif() +# Newer than VS .NET/VS Toolkit 2003 +set(_winsdk_msvc_greater_1310 OFF) +if(_WINDOWSSDK_IGNOREMSVC OR (MSVC AND (MSVC_VERSION GREATER 1310))) + set(_winsdk_msvc_greater_1310 ON) +endif() + +# VS2005/2008 +set(_winsdk_msvc_less_1600 OFF) +if(_WINDOWSSDK_IGNOREMSVC OR (MSVC AND (MSVC_VERSION LESS 1600))) + set(_winsdk_msvc_less_1600 ON) +endif() + +# VS2013+ +set(_winsdk_msvc_not_less_1800 OFF) +if(_WINDOWSSDK_IGNOREMSVC OR (MSVC AND (NOT MSVC_VERSION LESS 1800))) + set(_winsdk_msvc_not_less_1800 ON) +endif() + +### +# START body of find module +### +if(_winsdk_msvc_greater_1310) # Newer than VS .NET/VS Toolkit 2003 + ### + # Look for "preferred" SDKs + ### + + # Environment variable for SDK dir + if(EXISTS "$ENV{WindowsSDKDir}" AND (NOT "$ENV{WindowsSDKDir}" STREQUAL "")) + _winsdk_conditional_append_preferred("WindowsSDKDir environment variable" "$ENV{WindowsSDKDir}") + endif() + + if(_winsdk_msvc_less_1600) + # Per-user current Windows SDK for VS2005/2008 + get_filename_component(_sdkdir + "[HKEY_CURRENT_USER\\Software\\Microsoft\\Microsoft SDKs\\Windows;CurrentInstallFolder]" + ABSOLUTE) + _winsdk_conditional_append_preferred("Per-user current Windows SDK" "${_sdkdir}") + + # System-wide current Windows SDK for VS2005/2008 + get_filename_component(_sdkdir + "[HKEY_LOCAL_MACHINE\\SOFTWARE\\Microsoft\\Microsoft SDKs\\Windows;CurrentInstallFolder]" + ABSOLUTE) + _winsdk_conditional_append_preferred("System-wide current Windows SDK" "${_sdkdir}") + endif() + + ### + # Begin the massive list of SDK searching! + ### + if(_winsdk_vistaonly_ok AND _winsdk_msvc_not_less_1800) + # These require at least Visual Studio 2013 (VC12) + + _winsdk_check_microsoft_sdks_registry(v10.0A) + + # Windows Software Development Kit (SDK) for Windows 10 + # Several different versions living in the same directory - if nothing else we can assume RTM (10240) + _winsdk_check_microsoft_sdks_registry(v10.0 10.0.10240.0) + foreach(_win10build ${_winsdk_win10vers}) + _winsdk_check_win10_kits(${_win10build}) + endforeach() + endif() # vista-only and 2013+ + + # Included in Visual Studio 2013 + # Includes the v120_xp toolset + _winsdk_check_microsoft_sdks_registry(v8.1A 8.1.51636) + + if(_winsdk_vistaonly_ok AND _winsdk_msvc_not_less_1800) + # Windows Software Development Kit (SDK) for Windows 8.1 + # http://msdn.microsoft.com/en-gb/windows/desktop/bg162891 + _winsdk_check_microsoft_sdks_registry(v8.1 8.1.25984.0) + _winsdk_check_windows_kits_registry("Windows Kits 8.1" 8.1.25984.0 KitsRoot81) + endif() # vista-only and 2013+ + + if(_winsdk_vistaonly_ok) + # Included in Visual Studio 2012 + _winsdk_check_microsoft_sdks_registry(v8.0A 8.0.50727) + + # Microsoft Windows SDK for Windows 8 and .NET Framework 4.5 + # This is the first version to also include the DirectX SDK + # http://msdn.microsoft.com/en-US/windows/desktop/hh852363.aspx + _winsdk_check_microsoft_sdks_registry(v8.0 6.2.9200.16384) + _winsdk_check_windows_kits_registry("Windows Kits 8.0" 6.2.9200.16384 KitsRoot) + endif() # vista-only + + # Included with VS 2012 Update 1 or later + # Introduces v110_xp toolset + _winsdk_check_microsoft_sdks_registry(v7.1A 7.1.51106) + if(_winsdk_vistaonly_ok) + # Microsoft Windows SDK for Windows 7 and .NET Framework 4 + # http://www.microsoft.com/downloads/en/details.aspx?FamilyID=6b6c21d2-2006-4afa-9702-529fa782d63b + _winsdk_check_microsoft_sdks_registry(v7.1 7.1.7600.0.30514) + endif() # vista-only + + # Included with VS 2010 + _winsdk_check_microsoft_sdks_registry(v7.0A 6.1.7600.16385) + + # Windows SDK for Windows 7 and .NET Framework 3.5 SP1 + # Works with VC9 + # http://www.microsoft.com/en-us/download/details.aspx?id=18950 + _winsdk_check_microsoft_sdks_registry(v7.0 6.1.7600.16385) + + # Two versions call themselves "v6.1": + # Older: + # Windows Vista Update & .NET 3.0 SDK + # http://www.microsoft.com/en-us/download/details.aspx?id=14477 + + # Newer: + # Windows Server 2008 & .NET 3.5 SDK + # may have broken VS9SP1? they recommend v7.0 instead, or a KB... + # http://www.microsoft.com/en-us/download/details.aspx?id=24826 + _winsdk_check_microsoft_sdks_registry(v6.1 6.1.6000.16384.10) + + # Included in VS 2008 + _winsdk_check_microsoft_sdks_registry(v6.0A 6.1.6723.1) + + # Microsoft Windows Software Development Kit for Windows Vista and .NET Framework 3.0 Runtime Components + # http://blogs.msdn.com/b/stanley/archive/2006/11/08/microsoft-windows-software-development-kit-for-windows-vista-and-net-framework-3-0-runtime-components.aspx + _winsdk_check_microsoft_sdks_registry(v6.0 6.0.6000.16384) +endif() + +# Let's not forget the Platform SDKs, which sometimes are useful! +if(_winsdk_msvc_greater_1200) + _winsdk_check_platformsdk_registry("Microsoft Platform SDK for Windows Server 2003 R2" "5.2.3790.2075.51" "D2FF9F89-8AA2-4373-8A31-C838BF4DBBE1") + _winsdk_check_platformsdk_registry("Microsoft Platform SDK for Windows Server 2003 SP1" "5.2.3790.1830.15" "8F9E5EF3-A9A5-491B-A889-C58EFFECE8B3") +endif() +### +# Finally, look for "preferred" SDKs +### +if(_winsdk_msvc_greater_1310) # Newer than VS .NET/VS Toolkit 2003 + + + # Environment variable for SDK dir + if(EXISTS "$ENV{WindowsSDKDir}" AND (NOT "$ENV{WindowsSDKDir}" STREQUAL "")) + _winsdk_conditional_append_preferred("WindowsSDKDir environment variable" "$ENV{WindowsSDKDir}") + endif() + + if(_winsdk_msvc_less_1600) + # Per-user current Windows SDK for VS2005/2008 + get_filename_component(_sdkdir + "[HKEY_CURRENT_USER\\Software\\Microsoft\\Microsoft SDKs\\Windows;CurrentInstallFolder]" + ABSOLUTE) + _winsdk_conditional_append_preferred("Per-user current Windows SDK" "${_sdkdir}") + + # System-wide current Windows SDK for VS2005/2008 + get_filename_component(_sdkdir + "[HKEY_LOCAL_MACHINE\\SOFTWARE\\Microsoft\\Microsoft SDKs\\Windows;CurrentInstallFolder]" + ABSOLUTE) + _winsdk_conditional_append_preferred("System-wide current Windows SDK" "${_sdkdir}") + endif() +endif() + + +function(windowssdk_name_lookup _dir _outvar) + list(FIND _win_sdk_versanddirs "${_dir}" _diridx) + math(EXPR _idx "${_diridx} - 1") + if(${_idx} GREATER -1) + list(GET _win_sdk_versanddirs ${_idx} _ret) + else() + set(_ret "NOTFOUND") + endif() + set(${_outvar} "${_ret}" PARENT_SCOPE) +endfunction() + +function(windowssdk_build_lookup _dir _outvar) + list(FIND _win_sdk_buildsanddirs "${_dir}" _diridx) + math(EXPR _idx "${_diridx} - 1") + if(${_idx} GREATER -1) + list(GET _win_sdk_buildsanddirs ${_idx} _ret) + else() + set(_ret "NOTFOUND") + endif() + set(${_outvar} "${_ret}" PARENT_SCOPE) +endfunction() + +# If we found something... +if(_win_sdk_dirs) + list(GET _win_sdk_dirs 0 WINDOWSSDK_LATEST_DIR) + windowssdk_name_lookup("${WINDOWSSDK_LATEST_DIR}" + WINDOWSSDK_LATEST_NAME) + set(WINDOWSSDK_DIRS ${_win_sdk_dirs}) + + # Fallback, in case no preference found. + set(WINDOWSSDK_PREFERRED_DIR "${WINDOWSSDK_LATEST_DIR}") + set(WINDOWSSDK_PREFERRED_NAME "${WINDOWSSDK_LATEST_NAME}") + set(WINDOWSSDK_PREFERRED_FIRST_DIRS ${WINDOWSSDK_DIRS}) + set(WINDOWSSDK_FOUND_PREFERENCE OFF) +endif() + +# If we found indications of a user preference... +if(_win_sdk_preferred_sdk_dirs) + list(GET _win_sdk_preferred_sdk_dirs 0 WINDOWSSDK_PREFERRED_DIR) + windowssdk_name_lookup("${WINDOWSSDK_PREFERRED_DIR}" + WINDOWSSDK_PREFERRED_NAME) + set(WINDOWSSDK_PREFERRED_FIRST_DIRS + ${_win_sdk_preferred_sdk_dirs} + ${_win_sdk_dirs}) + list(REMOVE_DUPLICATES WINDOWSSDK_PREFERRED_FIRST_DIRS) + set(WINDOWSSDK_FOUND_PREFERENCE ON) +endif() + +include(FindPackageHandleStandardArgs) +find_package_handle_standard_args(WindowsSDK + "No compatible version of the Windows SDK or Platform SDK found." + WINDOWSSDK_DIRS) + +if(WINDOWSSDK_FOUND) + # Internal: Architecture-appropriate library directory names. + if("${CMAKE_VS_PLATFORM_NAME}" STREQUAL "ARM") + if(CMAKE_SIZEOF_VOID_P MATCHES "8") + # Only supported in Win10 SDK and up. + set(_winsdk_arch8 arm64) # what the WDK for Win8+ calls this architecture + else() + set(_winsdk_archbare /arm) # what the architecture used to be called in oldest SDKs + set(_winsdk_arch arm) # what the architecture used to be called + set(_winsdk_arch8 arm) # what the WDK for Win8+ calls this architecture + endif() + else() + if(CMAKE_SIZEOF_VOID_P MATCHES "8") + set(_winsdk_archbare /x64) # what the architecture used to be called in oldest SDKs + set(_winsdk_arch amd64) # what the architecture used to be called + set(_winsdk_arch8 x64) # what the WDK for Win8+ calls this architecture + else() + set(_winsdk_archbare ) # what the architecture used to be called in oldest SDKs + set(_winsdk_arch i386) # what the architecture used to be called + set(_winsdk_arch8 x86) # what the WDK for Win8+ calls this architecture + endif() + endif() + + function(get_windowssdk_from_component _component _var) + get_filename_component(_component "${_component}" ABSOLUTE) + file(TO_CMAKE_PATH "${_component}" _component) + foreach(_sdkdir ${WINDOWSSDK_DIRS}) + get_filename_component(_sdkdir "${_sdkdir}" ABSOLUTE) + string(LENGTH "${_sdkdir}" _sdklen) + file(RELATIVE_PATH _rel "${_sdkdir}" "${_component}") + # If we don't have any "parent directory" items... + if(NOT "${_rel}" MATCHES "[.][.]") + set(${_var} "${_sdkdir}" PARENT_SCOPE) + return() + endif() + endforeach() + # Fail. + set(${_var} "NOTFOUND" PARENT_SCOPE) + endfunction() + function(get_windowssdk_library_dirs _winsdk_dir _var) + set(_dirs) + set(_suffixes + "lib${_winsdk_archbare}" # SDKs like 7.1A + "lib/${_winsdk_arch}" # just because some SDKs have x86 dir and root dir + "lib/w2k/${_winsdk_arch}" # Win2k min requirement + "lib/wxp/${_winsdk_arch}" # WinXP min requirement + "lib/wnet/${_winsdk_arch}" # Win Server 2003 min requirement + "lib/wlh/${_winsdk_arch}" + "lib/wlh/um/${_winsdk_arch8}" # Win Vista ("Long Horn") min requirement + "lib/win7/${_winsdk_arch}" + "lib/win7/um/${_winsdk_arch8}" # Win 7 min requirement + ) + foreach(_ver + wlh # Win Vista ("Long Horn") min requirement + win7 # Win 7 min requirement + win8 # Win 8 min requirement + winv6.3 # Win 8.1 min requirement + ) + + list(APPEND _suffixes + "lib/${_ver}/${_winsdk_arch}" + "lib/${_ver}/um/${_winsdk_arch8}" + "lib/${_ver}/km/${_winsdk_arch8}" + ) + endforeach() + + # Look for WDF libraries in Win10+ SDK + foreach(_mode umdf kmdf) + file(GLOB _wdfdirs RELATIVE "${_winsdk_dir}" "${_winsdk_dir}/lib/wdf/${_mode}/${_winsdk_arch8}/*") + if(_wdfdirs) + list(APPEND _suffixes ${_wdfdirs}) + endif() + endforeach() + + # Look in each Win10+ SDK version for the components + foreach(_win10ver ${_winsdk_win10vers}) + foreach(_component um km ucrt mmos) + list(APPEND _suffixes "lib/${_win10ver}/${_component}/${_winsdk_arch8}") + endforeach() + endforeach() + + foreach(_suffix ${_suffixes}) + # Check to see if a library actually exists here. + file(GLOB _libs "${_winsdk_dir}/${_suffix}/*.lib") + if(_libs) + list(APPEND _dirs "${_winsdk_dir}/${_suffix}") + endif() + endforeach() + if("${_dirs}" STREQUAL "") + set(_dirs NOTFOUND) + else() + list(REMOVE_DUPLICATES _dirs) + endif() + set(${_var} ${_dirs} PARENT_SCOPE) + endfunction() + function(get_windowssdk_include_dirs _winsdk_dir _var) + set(_dirs) + + set(_subdirs shared um winrt km wdf mmos ucrt) + set(_suffixes Include) + + foreach(_dir ${_subdirs}) + list(APPEND _suffixes "Include/${_dir}") + endforeach() + + foreach(_ver ${_winsdk_win10vers}) + foreach(_dir ${_subdirs}) + list(APPEND _suffixes "Include/${_ver}/${_dir}") + endforeach() + endforeach() + + foreach(_suffix ${_suffixes}) + # Check to see if a header file actually exists here. + file(GLOB _headers "${_winsdk_dir}/${_suffix}/*.h") + if(_headers) + list(APPEND _dirs "${_winsdk_dir}/${_suffix}") + endif() + endforeach() + if("${_dirs}" STREQUAL "") + set(_dirs NOTFOUND) + else() + list(REMOVE_DUPLICATES _dirs) + endif() + set(${_var} ${_dirs} PARENT_SCOPE) + endfunction() + function(get_windowssdk_library_dirs_multiple _var) + set(_dirs) + foreach(_sdkdir ${ARGN}) + get_windowssdk_library_dirs("${_sdkdir}" _current_sdk_libdirs) + if(_current_sdk_libdirs) + list(APPEND _dirs ${_current_sdk_libdirs}) + endif() + endforeach() + if("${_dirs}" STREQUAL "") + set(_dirs NOTFOUND) + else() + list(REMOVE_DUPLICATES _dirs) + endif() + set(${_var} ${_dirs} PARENT_SCOPE) + endfunction() + function(get_windowssdk_include_dirs_multiple _var) + set(_dirs) + foreach(_sdkdir ${ARGN}) + get_windowssdk_include_dirs("${_sdkdir}" _current_sdk_incdirs) + if(_current_sdk_libdirs) + list(APPEND _dirs ${_current_sdk_incdirs}) + endif() + endforeach() + if("${_dirs}" STREQUAL "") + set(_dirs NOTFOUND) + else() + list(REMOVE_DUPLICATES _dirs) + endif() + set(${_var} ${_dirs} PARENT_SCOPE) + endfunction() +endif() diff --git a/src/cmake/Modules/GetGitRevisionDescription.cmake b/src/cmake/Modules/GetGitRevisionDescription.cmake index c8d27f2e8ce4..9f54191298b0 100644 --- a/src/cmake/Modules/GetGitRevisionDescription.cmake +++ b/src/cmake/Modules/GetGitRevisionDescription.cmake @@ -3,7 +3,7 @@ # These functions force a re-configure on each git commit so that you can # trust the values of the variables in your build system. # -# get_git_head_revision( [ ...]) +# get_git_head_revision( [ALLOW_LOOKING_ABOVE_CMAKE_SOURCE_DIR]) # # Returns the refspec and sha hash of the current head revision # @@ -12,26 +12,41 @@ # Returns the results of git describe on the source tree, and adjusting # the output so that it tests false if an error occurs. # +# git_describe_working_tree( [ ...]) +# +# Returns the results of git describe on the working tree (--dirty option), +# and adjusting the output so that it tests false if an error occurs. +# # git_get_exact_tag( [ ...]) # # Returns the results of git describe --exact-match on the source tree, # and adjusting the output so that it tests false if there was no exact # matching tag. # +# git_local_changes() +# +# Returns either "CLEAN" or "DIRTY" with respect to uncommitted changes. +# Uses the return code of "git diff-index --quiet HEAD --". +# Does not regard untracked files. +# # Requires CMake 2.6 or newer (uses the 'function' command) # # Original Author: -# 2009-2010 Ryan Pavlik -# http://academic.cleardefinition.com -# Iowa State University HCI Graduate Program/VRAC +# 2009-2020 Rylie Pavlik +# https://ryliepavlik.com/ +# +# Copyright 2009-2013, Iowa State University. +# Copyright 2013-2020, Rylie Pavlik +# Copyright 2013-2020, Contributors +# +# SPDX-License-Identifier: BSL-1.0 # -# Copyright Iowa State University 2009-2010. # Distributed under the Boost Software License, Version 1.0. # (See accompanying file LICENSE_1_0.txt or copy at # http://www.boost.org/LICENSE_1_0.txt) if(__get_git_revision_description) - return() + return() endif() set(__get_git_revision_description YES) @@ -39,92 +54,234 @@ set(__get_git_revision_description YES) # to find the path to this module rather than the path to a calling list file get_filename_component(_gitdescmoddir ${CMAKE_CURRENT_LIST_FILE} PATH) +# Function _git_find_closest_git_dir finds the next closest .git directory +# that is part of any directory in the path defined by _start_dir. +# The result is returned in the parent scope variable whose name is passed +# as variable _git_dir_var. If no .git directory can be found, the +# function returns an empty string via _git_dir_var. +# +# Example: Given a path C:/bla/foo/bar and assuming C:/bla/.git exists and +# neither foo nor bar contain a file/directory .git. This wil return +# C:/bla/.git +# +function(_git_find_closest_git_dir _start_dir _git_dir_var) + set(cur_dir "${_start_dir}") + set(git_dir "${_start_dir}/.git") + while(NOT EXISTS "${git_dir}") + # .git dir not found, search parent directories + set(git_previous_parent "${cur_dir}") + get_filename_component(cur_dir "${cur_dir}" DIRECTORY) + if(cur_dir STREQUAL git_previous_parent) + # We have reached the root directory, we are not in git + set(${_git_dir_var} + "" + PARENT_SCOPE) + return() + endif() + set(git_dir "${cur_dir}/.git") + endwhile() + set(${_git_dir_var} + "${git_dir}" + PARENT_SCOPE) +endfunction() + function(get_git_head_revision _refspecvar _hashvar) - set(GIT_PARENT_DIR "${CMAKE_CURRENT_SOURCE_DIR}") - set(GIT_DIR "${GIT_PARENT_DIR}/.git") - while(NOT EXISTS "${GIT_DIR}") # .git dir not found, search parent directories - set(GIT_PREVIOUS_PARENT "${GIT_PARENT_DIR}") - get_filename_component(GIT_PARENT_DIR ${GIT_PARENT_DIR} PATH) - if(GIT_PARENT_DIR STREQUAL GIT_PREVIOUS_PARENT) - # We have reached the root directory, we are not in git - set(${_refspecvar} "GITDIR-NOTFOUND" PARENT_SCOPE) - set(${_hashvar} "GITDIR-NOTFOUND" PARENT_SCOPE) - return() - endif() - set(GIT_DIR "${GIT_PARENT_DIR}/.git") - endwhile() - # check if this is a submodule - if(NOT IS_DIRECTORY ${GIT_DIR}) - file(READ ${GIT_DIR} submodule) - string(REGEX REPLACE "gitdir: (.*)\n$" "\\1" GIT_DIR_RELATIVE ${submodule}) - get_filename_component(SUBMODULE_DIR ${GIT_DIR} PATH) - get_filename_component(GIT_DIR ${SUBMODULE_DIR}/${GIT_DIR_RELATIVE} ABSOLUTE) - endif() - set(GIT_DATA "${CMAKE_CURRENT_BINARY_DIR}/CMakeFiles/git-data") - if(NOT EXISTS "${GIT_DATA}") - file(MAKE_DIRECTORY "${GIT_DATA}") - endif() - - if(NOT EXISTS "${GIT_DIR}/HEAD") - return() - endif() - set(HEAD_FILE "${GIT_DATA}/HEAD") - configure_file("${GIT_DIR}/HEAD" "${HEAD_FILE}" COPYONLY) - - configure_file("${_gitdescmoddir}/GetGitRevisionDescription.cmake.in" - "${GIT_DATA}/grabRef.cmake" - @ONLY) - include("${GIT_DATA}/grabRef.cmake") - - set(${_refspecvar} "${HEAD_REF}" PARENT_SCOPE) - set(${_hashvar} "${HEAD_HASH}" PARENT_SCOPE) + _git_find_closest_git_dir("${CMAKE_CURRENT_SOURCE_DIR}" GIT_DIR) + + if("${ARGN}" STREQUAL "ALLOW_LOOKING_ABOVE_CMAKE_SOURCE_DIR") + set(ALLOW_LOOKING_ABOVE_CMAKE_SOURCE_DIR TRUE) + else() + set(ALLOW_LOOKING_ABOVE_CMAKE_SOURCE_DIR FALSE) + endif() + if(NOT "${GIT_DIR}" STREQUAL "") + file(RELATIVE_PATH _relative_to_source_dir "${CMAKE_SOURCE_DIR}" + "${GIT_DIR}") + if("${_relative_to_source_dir}" MATCHES "[.][.]" + AND NOT ALLOW_LOOKING_ABOVE_CMAKE_SOURCE_DIR) + # We've gone above the CMake root dir. + set(GIT_DIR "") + endif() + endif() + if("${GIT_DIR}" STREQUAL "") + set(${_refspecvar} + "GITDIR-NOTFOUND" + PARENT_SCOPE) + set(${_hashvar} + "GITDIR-NOTFOUND" + PARENT_SCOPE) + return() + endif() + + # Check if the current source dir is a git submodule or a worktree. + # In both cases .git is a file instead of a directory. + # + if(NOT IS_DIRECTORY ${GIT_DIR}) + # The following git command will return a non empty string that + # points to the super project working tree if the current + # source dir is inside a git submodule. + # Otherwise the command will return an empty string. + # + execute_process( + COMMAND "${GIT_EXECUTABLE}" rev-parse + --show-superproject-working-tree + WORKING_DIRECTORY "${CMAKE_CURRENT_SOURCE_DIR}" + OUTPUT_VARIABLE out + ERROR_QUIET OUTPUT_STRIP_TRAILING_WHITESPACE) + if(NOT "${out}" STREQUAL "") + # If out is empty, GIT_DIR/CMAKE_CURRENT_SOURCE_DIR is in a submodule + file(READ ${GIT_DIR} submodule) + string(REGEX REPLACE "gitdir: (.*)$" "\\1" GIT_DIR_RELATIVE + ${submodule}) + string(STRIP ${GIT_DIR_RELATIVE} GIT_DIR_RELATIVE) + get_filename_component(SUBMODULE_DIR ${GIT_DIR} PATH) + get_filename_component(GIT_DIR ${SUBMODULE_DIR}/${GIT_DIR_RELATIVE} + ABSOLUTE) + set(HEAD_SOURCE_FILE "${GIT_DIR}/HEAD") + else() + # GIT_DIR/CMAKE_CURRENT_SOURCE_DIR is in a worktree + file(READ ${GIT_DIR} worktree_ref) + # The .git directory contains a path to the worktree information directory + # inside the parent git repo of the worktree. + # + string(REGEX REPLACE "gitdir: (.*)$" "\\1" git_worktree_dir + ${worktree_ref}) + string(STRIP ${git_worktree_dir} git_worktree_dir) + _git_find_closest_git_dir("${git_worktree_dir}" GIT_DIR) + set(HEAD_SOURCE_FILE "${git_worktree_dir}/HEAD") + endif() + else() + set(HEAD_SOURCE_FILE "${GIT_DIR}/HEAD") + endif() + set(GIT_DATA "${CMAKE_CURRENT_BINARY_DIR}/CMakeFiles/git-data") + if(NOT EXISTS "${GIT_DATA}") + file(MAKE_DIRECTORY "${GIT_DATA}") + endif() + + if(NOT EXISTS "${HEAD_SOURCE_FILE}") + return() + endif() + set(HEAD_FILE "${GIT_DATA}/HEAD") + configure_file("${HEAD_SOURCE_FILE}" "${HEAD_FILE}" COPYONLY) + + configure_file("${_gitdescmoddir}/GetGitRevisionDescription.cmake.in" + "${GIT_DATA}/grabRef.cmake" @ONLY) + include("${GIT_DATA}/grabRef.cmake") + + set(${_refspecvar} + "${HEAD_REF}" + PARENT_SCOPE) + set(${_hashvar} + "${HEAD_HASH}" + PARENT_SCOPE) endfunction() function(git_describe _var) - if(NOT GIT_FOUND) - find_package(Git QUIET) - endif() - get_git_head_revision(refspec hash) - if(NOT GIT_FOUND) - set(${_var} "GIT-NOTFOUND" PARENT_SCOPE) - return() - endif() - if(NOT hash) - set(${_var} "HEAD-HASH-NOTFOUND" PARENT_SCOPE) - return() - endif() - - # TODO sanitize - #if((${ARGN}" MATCHES "&&") OR - # (ARGN MATCHES "||") OR - # (ARGN MATCHES "\\;")) - # message("Please report the following error to the project!") - # message(FATAL_ERROR "Looks like someone's doing something nefarious with git_describe! Passed arguments ${ARGN}") - #endif() - - #message(STATUS "Arguments to execute_process: ${ARGN}") - - execute_process(COMMAND - "${GIT_EXECUTABLE}" - describe - ${hash} - ${ARGN} - WORKING_DIRECTORY - "${CMAKE_SOURCE_DIR}" - RESULT_VARIABLE - res - OUTPUT_VARIABLE - out - ERROR_QUIET - OUTPUT_STRIP_TRAILING_WHITESPACE) - if(NOT res EQUAL 0) - set(out "${out}-${res}-NOTFOUND") - endif() - - set(${_var} "${out}" PARENT_SCOPE) + if(NOT GIT_FOUND) + find_package(Git QUIET) + endif() + get_git_head_revision(refspec hash) + if(NOT GIT_FOUND) + set(${_var} + "GIT-NOTFOUND" + PARENT_SCOPE) + return() + endif() + if(NOT hash) + set(${_var} + "HEAD-HASH-NOTFOUND" + PARENT_SCOPE) + return() + endif() + + # TODO sanitize + #if((${ARGN}" MATCHES "&&") OR + # (ARGN MATCHES "||") OR + # (ARGN MATCHES "\\;")) + # message("Please report the following error to the project!") + # message(FATAL_ERROR "Looks like someone's doing something nefarious with git_describe! Passed arguments ${ARGN}") + #endif() + + #message(STATUS "Arguments to execute_process: ${ARGN}") + + execute_process( + COMMAND "${GIT_EXECUTABLE}" describe --tags --always ${hash} ${ARGN} + WORKING_DIRECTORY "${CMAKE_CURRENT_SOURCE_DIR}" + RESULT_VARIABLE res + OUTPUT_VARIABLE out + ERROR_QUIET OUTPUT_STRIP_TRAILING_WHITESPACE) + if(NOT res EQUAL 0) + set(out "${out}-${res}-NOTFOUND") + endif() + + set(${_var} + "${out}" + PARENT_SCOPE) +endfunction() + +function(git_describe_working_tree _var) + if(NOT GIT_FOUND) + find_package(Git QUIET) + endif() + if(NOT GIT_FOUND) + set(${_var} + "GIT-NOTFOUND" + PARENT_SCOPE) + return() + endif() + + execute_process( + COMMAND "${GIT_EXECUTABLE}" describe --dirty ${ARGN} + WORKING_DIRECTORY "${CMAKE_CURRENT_SOURCE_DIR}" + RESULT_VARIABLE res + OUTPUT_VARIABLE out + ERROR_QUIET OUTPUT_STRIP_TRAILING_WHITESPACE) + if(NOT res EQUAL 0) + set(out "${out}-${res}-NOTFOUND") + endif() + + set(${_var} + "${out}" + PARENT_SCOPE) endfunction() function(git_get_exact_tag _var) - git_describe(out --exact-match ${ARGN}) - set(${_var} "${out}" PARENT_SCOPE) + git_describe(out --exact-match ${ARGN}) + set(${_var} + "${out}" + PARENT_SCOPE) +endfunction() + +function(git_local_changes _var) + if(NOT GIT_FOUND) + find_package(Git QUIET) + endif() + get_git_head_revision(refspec hash) + if(NOT GIT_FOUND) + set(${_var} + "GIT-NOTFOUND" + PARENT_SCOPE) + return() + endif() + if(NOT hash) + set(${_var} + "HEAD-HASH-NOTFOUND" + PARENT_SCOPE) + return() + endif() + + execute_process( + COMMAND "${GIT_EXECUTABLE}" diff-index --quiet HEAD -- + WORKING_DIRECTORY "${CMAKE_CURRENT_SOURCE_DIR}" + RESULT_VARIABLE res + OUTPUT_VARIABLE out + ERROR_QUIET OUTPUT_STRIP_TRAILING_WHITESPACE) + if(res EQUAL 0) + set(${_var} + "CLEAN" + PARENT_SCOPE) + else() + set(${_var} + "DIRTY" + PARENT_SCOPE) + endif() endfunction() diff --git a/src/cmake/Modules/GetGitRevisionDescription.cmake.in b/src/cmake/Modules/GetGitRevisionDescription.cmake.in index 888ce13aaba3..9b8d20763759 100644 --- a/src/cmake/Modules/GetGitRevisionDescription.cmake.in +++ b/src/cmake/Modules/GetGitRevisionDescription.cmake.in @@ -1,17 +1,21 @@ -# +# # Internal file for GetGitRevisionDescription.cmake # # Requires CMake 2.6 or newer (uses the 'function' command) # # Original Author: -# 2009-2010 Ryan Pavlik -# http://academic.cleardefinition.com +# 2009-2023 Rylie Pavlik +# https://ryliepavlik.com/ # Iowa State University HCI Graduate Program/VRAC # -# Copyright Iowa State University 2009-2010. +# Copyright 2009-2012, Iowa State University +# Copyright 2011-2023, Contributors +# # Distributed under the Boost Software License, Version 1.0. # (See accompanying file LICENSE_1_0.txt or copy at # http://www.boost.org/LICENSE_1_0.txt) +# +# SPDX-License-Identifier: BSL-1.0 set(HEAD_HASH) @@ -19,20 +23,26 @@ file(READ "@HEAD_FILE@" HEAD_CONTENTS LIMIT 1024) string(STRIP "${HEAD_CONTENTS}" HEAD_CONTENTS) if(HEAD_CONTENTS MATCHES "ref") - # named branch - string(REPLACE "ref: " "" HEAD_REF "${HEAD_CONTENTS}") - if(EXISTS "@GIT_DIR@/${HEAD_REF}") - configure_file("@GIT_DIR@/${HEAD_REF}" "@GIT_DATA@/head-ref" COPYONLY) - elseif(EXISTS "@GIT_DIR@/logs/${HEAD_REF}") - configure_file("@GIT_DIR@/logs/${HEAD_REF}" "@GIT_DATA@/head-ref" COPYONLY) - set(HEAD_HASH "${HEAD_REF}") - endif() + # named branch + string(REPLACE "ref: " "" HEAD_REF "${HEAD_CONTENTS}") + if(EXISTS "@GIT_DIR@/${HEAD_REF}") + configure_file("@GIT_DIR@/${HEAD_REF}" "@GIT_DATA@/head-ref" COPYONLY) + else() + if(EXISTS "@GIT_DIR@/packed-refs") + configure_file("@GIT_DIR@/packed-refs" "@GIT_DATA@/packed-refs" + COPYONLY) + file(READ "@GIT_DATA@/packed-refs" PACKED_REFS) + if(${PACKED_REFS} MATCHES "([0-9a-z]*) ${HEAD_REF}") + set(HEAD_HASH "${CMAKE_MATCH_1}") + endif() + endif() + endif() else() - # detached HEAD - configure_file("@GIT_DIR@/HEAD" "@GIT_DATA@/head-ref" COPYONLY) + # detached HEAD + configure_file("@GIT_DIR@/HEAD" "@GIT_DATA@/head-ref" COPYONLY) endif() if(NOT HEAD_HASH) - file(READ "@GIT_DATA@/head-ref" HEAD_HASH LIMIT 1024) - string(STRIP "${HEAD_HASH}" HEAD_HASH) + file(READ "@GIT_DATA@/head-ref" HEAD_HASH LIMIT 1024) + string(STRIP "${HEAD_HASH}" HEAD_HASH) endif() diff --git a/src/cmake/Modules/README.md b/src/cmake/Modules/README.md new file mode 100644 index 000000000000..4d50b70d46d9 --- /dev/null +++ b/src/cmake/Modules/README.md @@ -0,0 +1,14 @@ +# CMake modules required for building Lean + +The files `GetGitRevisionDescription.cmake`, `GetGitRevisionDescription.cmake.in` and +`FindWindowsSDK.cmake` are part of the `cmake-modules` project by Rylie Pavlik. They +are licensed under the Boost Software License, Version 1.0. + +The modules should be updated when a new version of the Windows SDK is released. To do +so, obtain an up-to-date checkout of the `cmake-modules` project from +https://github.com/rpavlik/cmake-modules and run the following command from the root +of the `cmake-modules` repository: + +```bash +./update-modules.sh /path-to-lean4-repo/src/cmake/Modules +``` diff --git a/src/include/lean/lean.h b/src/include/lean/lean.h index c5a61269404f..a3b4a281d993 100644 --- a/src/include/lean/lean.h +++ b/src/include/lean/lean.h @@ -1847,6 +1847,140 @@ static inline uint8_t lean_usize_dec_le(size_t a1, size_t a2) { return a1 <= a2; static inline uint32_t lean_usize_to_uint32(size_t a) { return ((uint32_t)a); } static inline uint64_t lean_usize_to_uint64(size_t a) { return ((uint64_t)a); } +/* + * Note that we compile all files with -frwapv so in the following section all potential UB that + * may arise from signed overflow is forced to match 2's complement behavior. + * + * We furthermore rely on the implementation defined behavior of gcc/clang to apply reduction mod + * 2^N when casting to an integer type of size N: + * https://gcc.gnu.org/onlinedocs/gcc/Integers-implementation.html#Integers-implementation + * Unfortunately LLVM does not yet document their implementation defined behavior but it is + * most likely fine to rely on the fact that GCC and LLVM match on this: + * https://github.com/llvm/llvm-project/issues/11644 + */ + +/* Int8 */ +LEAN_EXPORT int8_t lean_int8_of_big_int(b_lean_obj_arg a); +static inline uint8_t lean_int8_of_int(b_lean_obj_arg a) { + int8_t res; + + if (lean_is_scalar(a)) { + res = (int8_t)lean_scalar_to_int64(a); + } else { + res = lean_int8_of_big_int(a); + } + + return (uint8_t)res; +} + +static inline lean_obj_res lean_int8_to_int(uint8_t a) { + int8_t arg = (int8_t)a; + return lean_int64_to_int((int64_t)arg); +} + +static inline uint8_t lean_int8_neg(uint8_t a) { + int8_t arg = (int8_t)a; + + return (uint8_t)(-arg); +} + +static inline uint8_t lean_int8_add(uint8_t a1, uint8_t a2) { + int8_t lhs = (int8_t) a1; + int8_t rhs = (int8_t) a2; + + return (uint8_t)(lhs + rhs); +} + +static inline uint8_t lean_int8_sub(uint8_t a1, uint8_t a2) { + int8_t lhs = (int8_t) a1; + int8_t rhs = (int8_t) a2; + + return (uint8_t)(lhs - rhs); +} + +static inline uint8_t lean_int8_mul(uint8_t a1, uint8_t a2) { + int8_t lhs = (int8_t) a1; + int8_t rhs = (int8_t) a2; + + return (uint8_t)(lhs * rhs); +} + +static inline uint8_t lean_int8_div(uint8_t a1, uint8_t a2) { + int8_t lhs = (int8_t) a1; + int8_t rhs = (int8_t) a2; + + return (uint8_t)(rhs == 0 ? 0 : lhs / rhs); +} + +static inline uint8_t lean_int8_mod(uint8_t a1, uint8_t a2) { + int8_t lhs = (int8_t) a1; + int8_t rhs = (int8_t) a2; + + return (uint8_t)(rhs == 0 ? 0 : lhs % rhs); +} + +static inline uint8_t lean_int8_land(uint8_t a1, uint8_t a2) { + int8_t lhs = (int8_t) a1; + int8_t rhs = (int8_t) a2; + + return (uint8_t)(lhs & rhs); +} + +static inline uint8_t lean_int8_lor(uint8_t a1, uint8_t a2) { + int8_t lhs = (int8_t) a1; + int8_t rhs = (int8_t) a2; + + return (uint8_t)(lhs | rhs); +} + +static inline uint8_t lean_int8_xor(uint8_t a1, uint8_t a2) { + int8_t lhs = (int8_t) a1; + int8_t rhs = (int8_t) a2; + + return (uint8_t)(lhs ^ rhs); +} + +static inline uint8_t lean_int8_shift_right(uint8_t a1, uint8_t a2) { + int8_t lhs = (int8_t) a1; + int8_t rhs = (int8_t) a2; + + return (uint8_t)(lhs >> (rhs % 8)); +} + +static inline uint8_t lean_int8_shift_left(uint8_t a1, uint8_t a2) { + int8_t lhs = (int8_t) a1; + int8_t rhs = (int8_t) a2; + + return (uint8_t)(lhs << (rhs % 8)); +} + +static inline uint8_t lean_int8_complement(uint8_t a) { + int8_t arg = (int8_t)a; + + return (uint8_t)(~arg); +} + +static inline uint8_t lean_int8_dec_eq(uint8_t a1, uint8_t a2) { + int8_t lhs = (int8_t) a1; + int8_t rhs = (int8_t) a2; + + return lhs == rhs; +} + +static inline uint8_t lean_int8_dec_lt(uint8_t a1, uint8_t a2) { + int8_t lhs = (int8_t) a1; + int8_t rhs = (int8_t) a2; + + return lhs < rhs; +} + +static inline uint8_t lean_int8_dec_le(uint8_t a1, uint8_t a2) { + int8_t lhs = (int8_t) a1; + int8_t rhs = (int8_t) a2; + + return lhs <= rhs; +} + /* Float */ LEAN_EXPORT lean_obj_res lean_float_to_string(double a); diff --git a/src/kernel/replace_fn.cpp b/src/kernel/replace_fn.cpp index 0a2b1030d12b..f97ef05cc630 100644 --- a/src/kernel/replace_fn.cpp +++ b/src/kernel/replace_fn.cpp @@ -12,6 +12,23 @@ Author: Leonardo de Moura namespace lean { +/* Like `is_exclusive`, but also consider unique MT references as unshared, which ensures we get + * similar performance on the cmdline and server (more precisely, for either option value of + * `internal.cmdlineSnapshots`). Note that as `e` is merely *borrowed* (e.g. from the mctx in + * the case of `instantiate_mvars` where the performance issue resolved here manifested, #5614), + * it is in fact possible that another thread could simultaneously add a new direct reference to + * `e`, so it is not definitely unshared in all cases if the below check is true. + * + * However, as we use this predicate merely as a conservative heuristic for detecting + * expressions that are unshared *within the expression tree* at hand, the approximation is + * still correct in this case. Furthermore, as we only use it for deciding when to cache + * results, it ultimately does not affect the correctness of the overall procedure in any case. + * This should however be kept in mind if we start using `is_likely_unshared` in other contexts. + */ +static bool is_likely_unshared(expr const & e) { + return e.raw()->m_rc == 1 || e.raw()->m_rc == -1; +} + class replace_rec_fn { struct key_hasher { std::size_t operator()(std::pair const & p) const { @@ -30,7 +47,7 @@ class replace_rec_fn { expr apply(expr const & e, unsigned offset) { bool shared = false; - if (m_use_cache && is_shared(e)) { + if (m_use_cache && !is_likely_unshared(e)) { auto it = m_cache.find(mk_pair(e.raw(), offset)); if (it != m_cache.end()) return it->second; diff --git a/src/runtime/hash.h b/src/runtime/hash.h index 4fcb70b8a682..105ec6ca67d3 100644 --- a/src/runtime/hash.h +++ b/src/runtime/hash.h @@ -6,7 +6,7 @@ Author: Leonardo de Moura */ #pragma once #include "runtime/debug.h" -#include "runtime/int64.h" +#include "runtime/int.h" namespace lean { diff --git a/src/runtime/int.h b/src/runtime/int.h new file mode 100644 index 000000000000..1163570244eb --- /dev/null +++ b/src/runtime/int.h @@ -0,0 +1,33 @@ +/* +Copyright (c) 2013 Microsoft Corporation. All rights reserved. +Released under Apache 2.0 license as described in the file LICENSE. + +Author: Leonardo de Moura +*/ +#include +#include +namespace lean { + +typedef int8_t int8; +typedef uint8_t uint8; +static_assert(sizeof(int8) == 1, "unexpected int8 size"); // NOLINT +static_assert(sizeof(uint8) == 1, "unexpected uint8 size"); // NOLINT + // +typedef int16_t int16; +typedef uint16_t uint16; +static_assert(sizeof(int16) == 2, "unexpected int16 size"); // NOLINT +static_assert(sizeof(uint16) == 2, "unexpected uint16 size"); // NOLINT + // +typedef int32_t int32; +typedef uint32_t uint32; +static_assert(sizeof(int32) == 4, "unexpected int32 size"); // NOLINT +static_assert(sizeof(uint32) == 4, "unexpected uint32 size"); // NOLINT + +typedef int64_t int64; +typedef uint64_t uint64; +static_assert(sizeof(int64) == 8, "unexpected int64 size"); // NOLINT +static_assert(sizeof(uint64) == 8, "unexpected uint64 size"); // NOLINT + // +typedef size_t usize; + +} diff --git a/src/runtime/int64.h b/src/runtime/int64.h deleted file mode 100644 index 47f6ef33dcbd..000000000000 --- a/src/runtime/int64.h +++ /dev/null @@ -1,13 +0,0 @@ -/* -Copyright (c) 2013 Microsoft Corporation. All rights reserved. -Released under Apache 2.0 license as described in the file LICENSE. - -Author: Leonardo de Moura -*/ -#include -namespace lean { -typedef int64_t int64; -typedef uint64_t uint64; -static_assert(sizeof(int64) == 8, "unexpected int64 size"); // NOLINT -static_assert(sizeof(uint64) == 8, "unexpected uint64 size"); // NOLINT -} diff --git a/src/runtime/mpz.cpp b/src/runtime/mpz.cpp index 8dc4a71c7d3c..b1d1af9e0d4e 100644 --- a/src/runtime/mpz.cpp +++ b/src/runtime/mpz.cpp @@ -239,22 +239,22 @@ void div2k(mpz & a, mpz const & b, unsigned k) { mpz_tdiv_q_2exp(a.m_val, b.m_val, k); } -unsigned mpz::mod8() const { +uint8 mpz::mod8() const { mpz a; mpz_tdiv_r_2exp(a.m_val, m_val, 8); - return a.get_unsigned_int(); + return static_cast(a.get_unsigned_int()); } -unsigned mpz::mod16() const { +uint16 mpz::mod16() const { mpz a; mpz_tdiv_r_2exp(a.m_val, m_val, 16); - return a.get_unsigned_int(); + return static_cast(a.get_unsigned_int()); } -unsigned mpz::mod32() const { +uint32 mpz::mod32() const { mpz a; mpz_tdiv_r_2exp(a.m_val, m_val, 32); - return a.get_unsigned_int(); + return static_cast(a.get_unsigned_int()); } uint64 mpz::mod64() const { @@ -267,6 +267,12 @@ uint64 mpz::mod64() const { return (static_cast(h.get_unsigned_int()) << 32) + static_cast(l.get_unsigned_int()); } +int8 mpz::smod8() const { + mpz a; + mpz_tdiv_r_2exp(a.m_val, m_val, 8); + return static_cast(a.get_int()); +} + void power(mpz & a, mpz const & b, unsigned k) { mpz_pow_ui(a.m_val, b.m_val, k); } @@ -945,16 +951,16 @@ void div2k(mpz & a, mpz const & b, unsigned k) { a.set(new_sz, ds.begin()); } -unsigned mpz::mod8() const { - return m_digits[0] & 0xFFu; +uint8 mpz::mod8() const { + return static_cast(m_digits[0] & 0xFFu); } -unsigned mpz::mod16() const { - return m_digits[0] & 0xFFFFu; +uint16 mpz::mod16() const { + return static_cast(m_digits[0] & 0xFFFFu); } -unsigned mpz::mod32() const { - return m_digits[0]; +uint32 mpz::mod32() const { + return static_cast(m_digits[0]); } uint64 mpz::mod64() const { @@ -964,6 +970,14 @@ uint64 mpz::mod64() const { return m_digits[0] + (static_cast(m_digits[1]) << 8*sizeof(mpn_digit)); } +int8 mpz::smod8() const { + int8_t val = mod8(); + if (m_sign) { + val = -val; + } + return val; +} + void power(mpz & a, mpz const & b, unsigned k) { a = b; a.pow(k); diff --git a/src/runtime/mpz.h b/src/runtime/mpz.h index 68127c4606fd..82f1a283dcb4 100644 --- a/src/runtime/mpz.h +++ b/src/runtime/mpz.h @@ -15,7 +15,7 @@ Author: Leonardo de Moura #include #include #include -#include "runtime/int64.h" +#include "runtime/int.h" #include "runtime/debug.h" namespace lean { @@ -266,11 +266,13 @@ class LEAN_EXPORT mpz { // a <- b / 2^k friend void div2k(mpz & a, mpz const & b, unsigned k); - unsigned mod8() const; - unsigned mod16() const; - unsigned mod32() const; + uint8 mod8() const; + uint16 mod16() const; + uint32 mod32() const; uint64 mod64() const; + int8 smod8() const; + /** \brief Return the position of the most significant bit. Return 0 if the number is negative diff --git a/src/runtime/object.cpp b/src/runtime/object.cpp index eb6461f7cf8f..8d0f59c47914 100644 --- a/src/runtime/object.cpp +++ b/src/runtime/object.cpp @@ -1536,11 +1536,11 @@ extern "C" LEAN_EXPORT bool lean_int_big_nonneg(object * a) { // UInt extern "C" LEAN_EXPORT uint8 lean_uint8_of_big_nat(b_obj_arg a) { - return static_cast(mpz_value(a).mod8()); + return mpz_value(a).mod8(); } extern "C" LEAN_EXPORT uint16 lean_uint16_of_big_nat(b_obj_arg a) { - return static_cast(mpz_value(a).mod16()); + return mpz_value(a).mod16(); } extern "C" LEAN_EXPORT uint32 lean_uint32_of_big_nat(b_obj_arg a) { @@ -1574,6 +1574,13 @@ extern "C" LEAN_EXPORT usize lean_usize_big_modn(usize a1, b_lean_obj_arg) { return a1; } +// ======================================= +// IntX + +extern "C" LEAN_EXPORT int8 lean_int8_of_big_int(b_obj_arg a) { + return mpz_value(a).smod8(); +} + // ======================================= // Float diff --git a/src/runtime/object.h b/src/runtime/object.h index b5e5a6375817..24ebe298a595 100644 --- a/src/runtime/object.h +++ b/src/runtime/object.h @@ -10,11 +10,6 @@ Author: Leonardo de Moura #include "runtime/mpz.h" namespace lean { -typedef uint8_t uint8; -typedef uint16_t uint16; -typedef uint32_t uint32; -typedef uint64_t uint64; -typedef size_t usize; typedef lean_object object; typedef object * obj_arg; diff --git a/src/util/message_definitions.h b/src/util/message_definitions.h index 94aa8cf65990..53426634ffa3 100644 --- a/src/util/message_definitions.h +++ b/src/util/message_definitions.h @@ -7,7 +7,7 @@ Author: Gabriel Ebner #pragma once #include #include -#include "runtime/int64.h" +#include "runtime/int.h" #include "util/name.h" namespace lean { diff --git a/stage0/src/CMakeLists.txt b/stage0/src/CMakeLists.txt index 2b36ee213b2c..56b9bf8bd410 100644 --- a/stage0/src/CMakeLists.txt +++ b/stage0/src/CMakeLists.txt @@ -155,6 +155,10 @@ endif () # We want explicit stack probes in huge Lean stack frames for robust stack overflow detection string(APPEND LEANC_EXTRA_FLAGS " -fstack-clash-protection") +# This makes signed integer overflow guaranteed to match 2's complement. +string(APPEND CMAKE_CXX_FLAGS " -fwrapv") +string(APPEND LEANC_EXTRA_FLAGS " -fwrapv") + if(NOT MULTI_THREAD) message(STATUS "Disabled multi-thread support, it will not be safe to run multiple threads in parallel") set(AUTO_THREAD_FINALIZATION OFF) @@ -297,6 +301,23 @@ if(NOT LEAN_STANDALONE) string(APPEND LEAN_EXTRA_LINKER_FLAGS " ${LIBUV_LIBRARIES}") endif() +# Windows SDK (for ICU) +if(${CMAKE_SYSTEM_NAME} MATCHES "Windows") + # Pass 'tools' to skip MSVC version check (as MSVC/Visual Studio is not necessarily installed) + find_package(WindowsSDK REQUIRED COMPONENTS tools) + + # This will give a semicolon-separated list of include directories + get_windowssdk_include_dirs(${WINDOWSSDK_LATEST_DIR} WINDOWSSDK_INCLUDE_DIRS) + + # To successfully build against Windows SDK headers, the Windows SDK headers must have lower + # priority than other system headers, so use `-idirafter`. Unfortunately, CMake does not + # support this using `include_directories`. + string(REPLACE ";" "\" -idirafter \"" WINDOWSSDK_INCLUDE_DIRS "${WINDOWSSDK_INCLUDE_DIRS}") + string(APPEND CMAKE_CXX_FLAGS " -idirafter \"${WINDOWSSDK_INCLUDE_DIRS}\"") + + string(APPEND LEAN_EXTRA_LINKER_FLAGS " -licu") +endif() + # ccache if(CCACHE AND NOT CMAKE_CXX_COMPILER_LAUNCHER AND NOT CMAKE_C_COMPILER_LAUNCHER) find_program(CCACHE_PATH ccache) @@ -480,7 +501,7 @@ endif() # Git HASH if(USE_GITHASH) include(GetGitRevisionDescription) - get_git_head_revision(GIT_REFSPEC GIT_SHA1) + get_git_head_revision(GIT_REFSPEC GIT_SHA1 ALLOW_LOOKING_ABOVE_CMAKE_SOURCE_DIR) if(${GIT_SHA1} MATCHES "GITDIR-NOTFOUND") message(STATUS "Failed to read git_sha1") set(GIT_SHA1 "") diff --git a/stage0/src/cmake/Modules/FindWindowsSDK.cmake b/stage0/src/cmake/Modules/FindWindowsSDK.cmake new file mode 100644 index 000000000000..17519ba59b18 --- /dev/null +++ b/stage0/src/cmake/Modules/FindWindowsSDK.cmake @@ -0,0 +1,643 @@ +# - Find the Windows SDK aka Platform SDK +# +# Relevant Wikipedia article: http://en.wikipedia.org/wiki/Microsoft_Windows_SDK +# +# Pass "COMPONENTS tools" to ignore Visual Studio version checks: in case +# you just want the tool binaries to run, rather than the libraries and headers +# for compiling. +# +# Variables: +# WINDOWSSDK_FOUND - if any version of the windows or platform SDK was found that is usable with the current version of visual studio +# WINDOWSSDK_LATEST_DIR +# WINDOWSSDK_LATEST_NAME +# WINDOWSSDK_FOUND_PREFERENCE - if we found an entry indicating a "preferred" SDK listed for this visual studio version +# WINDOWSSDK_PREFERRED_DIR +# WINDOWSSDK_PREFERRED_NAME +# +# WINDOWSSDK_DIRS - contains no duplicates, ordered most recent first. +# WINDOWSSDK_PREFERRED_FIRST_DIRS - contains no duplicates, ordered with preferred first, followed by the rest in descending recency +# +# Functions: +# windowssdk_name_lookup( ) - Find the name corresponding with the SDK directory you pass in, or +# NOTFOUND if not recognized. Your directory must be one of WINDOWSSDK_DIRS for this to work. +# +# windowssdk_build_lookup( ) - Find the build version number corresponding with the SDK directory you pass in, or +# NOTFOUND if not recognized. Your directory must be one of WINDOWSSDK_DIRS for this to work. +# +# get_windowssdk_from_component( ) - Given a library or include dir, +# find the Windows SDK root dir corresponding to it, or NOTFOUND if unrecognized. +# +# get_windowssdk_library_dirs( ) - Find the architecture-appropriate +# library directories corresponding to the SDK directory you pass in (or NOTFOUND if none) +# +# get_windowssdk_library_dirs_multiple( ...) - Find the architecture-appropriate +# library directories corresponding to the SDK directories you pass in, in order, skipping those not found. NOTFOUND if none at all. +# Good for passing WINDOWSSDK_DIRS or WINDOWSSDK_DIRS to if you really just want a file and don't care where from. +# +# get_windowssdk_include_dirs( ) - Find the +# include directories corresponding to the SDK directory you pass in (or NOTFOUND if none) +# +# get_windowssdk_include_dirs_multiple( ...) - Find the +# include directories corresponding to the SDK directories you pass in, in order, skipping those not found. NOTFOUND if none at all. +# Good for passing WINDOWSSDK_DIRS or WINDOWSSDK_DIRS to if you really just want a file and don't care where from. +# +# Requires these CMake modules: +# FindPackageHandleStandardArgs (known included with CMake >=2.6.2) +# +# Original Author: +# 2012 Rylie Pavlik +# https://ryliepavlik.com/ +# Iowa State University HCI Graduate Program/VRAC +# +# Copyright 2012, Iowa State University +# +# Distributed under the Boost Software License, Version 1.0. +# (See accompanying file LICENSE_1_0.txt or copy at +# http://www.boost.org/LICENSE_1_0.txt) +# +# SPDX-License-Identifier: BSL-1.0 + +set(_preferred_sdk_dirs) # pre-output +set(_win_sdk_dirs) # pre-output +set(_win_sdk_versanddirs) # pre-output +set(_win_sdk_buildsanddirs) # pre-output +set(_winsdk_vistaonly) # search parameters +set(_winsdk_kits) # search parameters + + +set(_WINDOWSSDK_ANNOUNCE OFF) +if(NOT WINDOWSSDK_FOUND AND (NOT WindowsSDK_FIND_QUIETLY)) + set(_WINDOWSSDK_ANNOUNCE ON) +endif() +macro(_winsdk_announce) + if(_WINSDK_ANNOUNCE) + message(STATUS ${ARGN}) + endif() +endmacro() + +# See https://developer.microsoft.com/en-us/windows/downloads/sdk-archive - +# although version numbers listed on that page don't necessarily match the directory +# used by the installer. +set(_winsdk_win10vers + 10.0.26100.0 + 10.0.22621.0 + 10.0.22000.0 + 10.0.20348.0 + 10.0.19041.0 + 10.0.18362.0 # Win10 1903 "19H1" + 10.0.17763.0 # Win10 1809 "October 2018 Update" + 10.0.17134.0 # Redstone 4 aka Win10 1803 "April 2018 Update" + 10.0.17133.0 # Redstone 4 aka Win10 1803 "April 2018 Update" + 10.0.16299.0 # Redstone 3 aka Win10 1709 "Fall Creators Update" + 10.0.15063.0 # Redstone 2 aka Win10 1703 "Creators Update" + 10.0.14393.0 # Redstone aka Win10 1607 "Anniversary Update" + 10.0.10586.0 # TH2 aka Win10 1511 + 10.0.10240.0 # Win10 RTM + 10.0.10150.0 # just ucrt + 10.0.10056.0 +) + +if(WindowsSDK_FIND_COMPONENTS MATCHES "tools") + set(_WINDOWSSDK_IGNOREMSVC ON) + _winsdk_announce("Checking for tools from Windows/Platform SDKs...") +else() + set(_WINDOWSSDK_IGNOREMSVC OFF) + _winsdk_announce("Checking for Windows/Platform SDKs...") +endif() + +# Appends to the three main pre-output lists used only if the path exists +# and is not already in the list. +function(_winsdk_conditional_append _vername _build _path) + if(("${_path}" MATCHES "registry") OR (NOT EXISTS "${_path}")) + # Path invalid - do not add + return() + endif() + list(FIND _win_sdk_dirs "${_path}" _win_sdk_idx) + if(_win_sdk_idx GREATER -1) + # Path already in list - do not add + return() + endif() + _winsdk_announce( " - ${_vername}, Build ${_build} @ ${_path}") + # Not yet in the list, so we'll add it + list(APPEND _win_sdk_dirs "${_path}") + set(_win_sdk_dirs "${_win_sdk_dirs}" CACHE INTERNAL "" FORCE) + list(APPEND + _win_sdk_versanddirs + "${_vername}" + "${_path}") + set(_win_sdk_versanddirs "${_win_sdk_versanddirs}" CACHE INTERNAL "" FORCE) + list(APPEND + _win_sdk_buildsanddirs + "${_build}" + "${_path}") + set(_win_sdk_buildsanddirs "${_win_sdk_buildsanddirs}" CACHE INTERNAL "" FORCE) +endfunction() + +# Appends to the "preferred SDK" lists only if the path exists +function(_winsdk_conditional_append_preferred _info _path) + if(("${_path}" MATCHES "registry") OR (NOT EXISTS "${_path}")) + # Path invalid - do not add + return() + endif() + + get_filename_component(_path "${_path}" ABSOLUTE) + + list(FIND _win_sdk_preferred_sdk_dirs "${_path}" _win_sdk_idx) + if(_win_sdk_idx GREATER -1) + # Path already in list - do not add + return() + endif() + _winsdk_announce( " - Found \"preferred\" SDK ${_info} @ ${_path}") + # Not yet in the list, so we'll add it + list(APPEND _win_sdk_preferred_sdk_dirs "${_path}") + set(_win_sdk_preferred_sdk_dirs "${_win_sdk_dirs}" CACHE INTERNAL "" FORCE) + + # Just in case we somehow missed it: + _winsdk_conditional_append("${_info}" "" "${_path}") +endfunction() + +# Given a version like v7.0A, looks for an SDK in the registry under "Microsoft SDKs". +# If the given version might be in both HKEY_LOCAL_MACHINE\\SOFTWARE\\Microsoft\\Microsoft SDKs\\Windows +# and HKEY_LOCAL_MACHINE\\SOFTWARE\\Microsoft\\Windows Kits\\Installed Roots aka "Windows Kits", +# use this macro first, since these registry keys usually have more information. +# +# Pass a "default" build number as an extra argument in case we can't find it. +function(_winsdk_check_microsoft_sdks_registry _winsdkver) + set(SDKKEY "HKEY_LOCAL_MACHINE\\SOFTWARE\\Microsoft\\Microsoft SDKs\\Windows\\${_winsdkver}") + get_filename_component(_sdkdir + "[${SDKKEY};InstallationFolder]" + ABSOLUTE) + + set(_sdkname "Windows SDK ${_winsdkver}") + + # Default build number passed as extra argument + set(_build ${ARGN}) + # See if the registry holds a Microsoft-mutilated, err, designated, product name + # (just using get_filename_component to execute the registry lookup) + get_filename_component(_sdkproductname + "[${SDKKEY};ProductName]" + NAME) + if(NOT "${_sdkproductname}" MATCHES "registry") + # Got a product name + set(_sdkname "${_sdkname} (${_sdkproductname})") + endif() + + # try for a version to augment our name + # (just using get_filename_component to execute the registry lookup) + get_filename_component(_sdkver + "[${SDKKEY};ProductVersion]" + NAME) + if(NOT "${_sdkver}" MATCHES "registry" AND NOT MATCHES) + # Got a version + if(NOT "${_sdkver}" MATCHES "\\.\\.") + # and it's not an invalid one with two dots in it: + # use to override the default build + set(_build ${_sdkver}) + if(NOT "${_sdkname}" MATCHES "${_sdkver}") + # Got a version that's not already in the name, let's use it to improve our name. + set(_sdkname "${_sdkname} (${_sdkver})") + endif() + endif() + endif() + _winsdk_conditional_append("${_sdkname}" "${_build}" "${_sdkdir}") +endfunction() + +# Given a name for identification purposes, the build number, and a key (technically a "value name") +# corresponding to a Windows SDK packaged as a "Windows Kit", look for it +# in HKEY_LOCAL_MACHINE\\SOFTWARE\\Microsoft\\Windows Kits\\Installed Roots +# Note that the key or "value name" tends to be something weird like KitsRoot81 - +# no easy way to predict, just have to observe them in the wild. +# Doesn't hurt to also try _winsdk_check_microsoft_sdks_registry for these: +# sometimes you get keys in both parts of the registry (in the wow64 portion especially), +# and the non-"Windows Kits" location is often more descriptive. +function(_winsdk_check_windows_kits_registry _winkit_name _winkit_build _winkit_key) + get_filename_component(_sdkdir + "[HKEY_LOCAL_MACHINE\\SOFTWARE\\Microsoft\\Windows Kits\\Installed Roots;${_winkit_key}]" + ABSOLUTE) + _winsdk_conditional_append("${_winkit_name}" "${_winkit_build}" "${_sdkdir}") +endfunction() + +# Given a name for identification purposes and the build number +# corresponding to a Windows 10 SDK packaged as a "Windows Kit", look for it +# in HKEY_LOCAL_MACHINE\\SOFTWARE\\Microsoft\\Windows Kits\\Installed Roots +# Doesn't hurt to also try _winsdk_check_microsoft_sdks_registry for these: +# sometimes you get keys in both parts of the registry (in the wow64 portion especially), +# and the non-"Windows Kits" location is often more descriptive. +function(_winsdk_check_win10_kits _winkit_build) + get_filename_component(_sdkdir + "[HKEY_LOCAL_MACHINE\\SOFTWARE\\Microsoft\\Windows Kits\\Installed Roots;KitsRoot10]" + ABSOLUTE) + if(("${_sdkdir}" MATCHES "registry") OR (NOT EXISTS "${_sdkdir}")) + return() # not found + endif() + if(EXISTS "${_sdkdir}/Include/${_winkit_build}/um") + _winsdk_conditional_append("Windows Kits 10 (Build ${_winkit_build})" "${_winkit_build}" "${_sdkdir}") + endif() +endfunction() + +# Given a name for indentification purposes, the build number, and the associated package GUID, +# look in the registry under both HKLM and HKCU in \\SOFTWARE\\Microsoft\\MicrosoftSDK\\InstalledSDKs\\ +# for that guid and the SDK it points to. +function(_winsdk_check_platformsdk_registry _platformsdkname _build _platformsdkguid) + foreach(_winsdk_hive HKEY_LOCAL_MACHINE HKEY_CURRENT_USER) + get_filename_component(_sdkdir + "[${_winsdk_hive}\\SOFTWARE\\Microsoft\\MicrosoftSDK\\InstalledSDKs\\${_platformsdkguid};Install Dir]" + ABSOLUTE) + _winsdk_conditional_append("${_platformsdkname} (${_build})" "${_build}" "${_sdkdir}") + endforeach() +endfunction() + +### +# Detect toolchain information: to know whether it's OK to use Vista+ only SDKs +### +set(_winsdk_vistaonly_ok OFF) +if(MSVC AND NOT _WINDOWSSDK_IGNOREMSVC) + # VC 10 and older has broad target support + if(MSVC_VERSION LESS 1700) + # VC 11 by default targets Vista and later only, so we can add a few more SDKs that (might?) only work on vista+ + elseif("${CMAKE_VS_PLATFORM_TOOLSET}" MATCHES "_xp") + # This is the XP-compatible v110+ toolset + elseif("${CMAKE_VS_PLATFORM_TOOLSET}" STREQUAL "v100" OR "${CMAKE_VS_PLATFORM_TOOLSET}" STREQUAL "v90") + # This is the VS2010/VS2008 toolset + else() + # OK, we're VC11 or newer and not using a backlevel or XP-compatible toolset. + # These versions have no XP (and possibly Vista pre-SP1) support + set(_winsdk_vistaonly_ok ON) + if(_WINDOWSSDK_ANNOUNCE AND NOT _WINDOWSSDK_VISTAONLY_PESTERED) + set(_WINDOWSSDK_VISTAONLY_PESTERED ON CACHE INTERNAL "" FORCE) + message(STATUS "FindWindowsSDK: Detected Visual Studio 2012 or newer, not using the _xp toolset variant: including SDK versions that drop XP support in search!") + endif() + endif() +endif() +if(_WINDOWSSDK_IGNOREMSVC) + set(_winsdk_vistaonly_ok ON) +endif() + +### +# MSVC version checks - keeps messy conditionals in one place +# (messy because of _WINDOWSSDK_IGNOREMSVC) +### +set(_winsdk_msvc_greater_1200 OFF) +if(_WINDOWSSDK_IGNOREMSVC OR (MSVC AND (MSVC_VERSION GREATER 1200))) + set(_winsdk_msvc_greater_1200 ON) +endif() +# Newer than VS .NET/VS Toolkit 2003 +set(_winsdk_msvc_greater_1310 OFF) +if(_WINDOWSSDK_IGNOREMSVC OR (MSVC AND (MSVC_VERSION GREATER 1310))) + set(_winsdk_msvc_greater_1310 ON) +endif() + +# VS2005/2008 +set(_winsdk_msvc_less_1600 OFF) +if(_WINDOWSSDK_IGNOREMSVC OR (MSVC AND (MSVC_VERSION LESS 1600))) + set(_winsdk_msvc_less_1600 ON) +endif() + +# VS2013+ +set(_winsdk_msvc_not_less_1800 OFF) +if(_WINDOWSSDK_IGNOREMSVC OR (MSVC AND (NOT MSVC_VERSION LESS 1800))) + set(_winsdk_msvc_not_less_1800 ON) +endif() + +### +# START body of find module +### +if(_winsdk_msvc_greater_1310) # Newer than VS .NET/VS Toolkit 2003 + ### + # Look for "preferred" SDKs + ### + + # Environment variable for SDK dir + if(EXISTS "$ENV{WindowsSDKDir}" AND (NOT "$ENV{WindowsSDKDir}" STREQUAL "")) + _winsdk_conditional_append_preferred("WindowsSDKDir environment variable" "$ENV{WindowsSDKDir}") + endif() + + if(_winsdk_msvc_less_1600) + # Per-user current Windows SDK for VS2005/2008 + get_filename_component(_sdkdir + "[HKEY_CURRENT_USER\\Software\\Microsoft\\Microsoft SDKs\\Windows;CurrentInstallFolder]" + ABSOLUTE) + _winsdk_conditional_append_preferred("Per-user current Windows SDK" "${_sdkdir}") + + # System-wide current Windows SDK for VS2005/2008 + get_filename_component(_sdkdir + "[HKEY_LOCAL_MACHINE\\SOFTWARE\\Microsoft\\Microsoft SDKs\\Windows;CurrentInstallFolder]" + ABSOLUTE) + _winsdk_conditional_append_preferred("System-wide current Windows SDK" "${_sdkdir}") + endif() + + ### + # Begin the massive list of SDK searching! + ### + if(_winsdk_vistaonly_ok AND _winsdk_msvc_not_less_1800) + # These require at least Visual Studio 2013 (VC12) + + _winsdk_check_microsoft_sdks_registry(v10.0A) + + # Windows Software Development Kit (SDK) for Windows 10 + # Several different versions living in the same directory - if nothing else we can assume RTM (10240) + _winsdk_check_microsoft_sdks_registry(v10.0 10.0.10240.0) + foreach(_win10build ${_winsdk_win10vers}) + _winsdk_check_win10_kits(${_win10build}) + endforeach() + endif() # vista-only and 2013+ + + # Included in Visual Studio 2013 + # Includes the v120_xp toolset + _winsdk_check_microsoft_sdks_registry(v8.1A 8.1.51636) + + if(_winsdk_vistaonly_ok AND _winsdk_msvc_not_less_1800) + # Windows Software Development Kit (SDK) for Windows 8.1 + # http://msdn.microsoft.com/en-gb/windows/desktop/bg162891 + _winsdk_check_microsoft_sdks_registry(v8.1 8.1.25984.0) + _winsdk_check_windows_kits_registry("Windows Kits 8.1" 8.1.25984.0 KitsRoot81) + endif() # vista-only and 2013+ + + if(_winsdk_vistaonly_ok) + # Included in Visual Studio 2012 + _winsdk_check_microsoft_sdks_registry(v8.0A 8.0.50727) + + # Microsoft Windows SDK for Windows 8 and .NET Framework 4.5 + # This is the first version to also include the DirectX SDK + # http://msdn.microsoft.com/en-US/windows/desktop/hh852363.aspx + _winsdk_check_microsoft_sdks_registry(v8.0 6.2.9200.16384) + _winsdk_check_windows_kits_registry("Windows Kits 8.0" 6.2.9200.16384 KitsRoot) + endif() # vista-only + + # Included with VS 2012 Update 1 or later + # Introduces v110_xp toolset + _winsdk_check_microsoft_sdks_registry(v7.1A 7.1.51106) + if(_winsdk_vistaonly_ok) + # Microsoft Windows SDK for Windows 7 and .NET Framework 4 + # http://www.microsoft.com/downloads/en/details.aspx?FamilyID=6b6c21d2-2006-4afa-9702-529fa782d63b + _winsdk_check_microsoft_sdks_registry(v7.1 7.1.7600.0.30514) + endif() # vista-only + + # Included with VS 2010 + _winsdk_check_microsoft_sdks_registry(v7.0A 6.1.7600.16385) + + # Windows SDK for Windows 7 and .NET Framework 3.5 SP1 + # Works with VC9 + # http://www.microsoft.com/en-us/download/details.aspx?id=18950 + _winsdk_check_microsoft_sdks_registry(v7.0 6.1.7600.16385) + + # Two versions call themselves "v6.1": + # Older: + # Windows Vista Update & .NET 3.0 SDK + # http://www.microsoft.com/en-us/download/details.aspx?id=14477 + + # Newer: + # Windows Server 2008 & .NET 3.5 SDK + # may have broken VS9SP1? they recommend v7.0 instead, or a KB... + # http://www.microsoft.com/en-us/download/details.aspx?id=24826 + _winsdk_check_microsoft_sdks_registry(v6.1 6.1.6000.16384.10) + + # Included in VS 2008 + _winsdk_check_microsoft_sdks_registry(v6.0A 6.1.6723.1) + + # Microsoft Windows Software Development Kit for Windows Vista and .NET Framework 3.0 Runtime Components + # http://blogs.msdn.com/b/stanley/archive/2006/11/08/microsoft-windows-software-development-kit-for-windows-vista-and-net-framework-3-0-runtime-components.aspx + _winsdk_check_microsoft_sdks_registry(v6.0 6.0.6000.16384) +endif() + +# Let's not forget the Platform SDKs, which sometimes are useful! +if(_winsdk_msvc_greater_1200) + _winsdk_check_platformsdk_registry("Microsoft Platform SDK for Windows Server 2003 R2" "5.2.3790.2075.51" "D2FF9F89-8AA2-4373-8A31-C838BF4DBBE1") + _winsdk_check_platformsdk_registry("Microsoft Platform SDK for Windows Server 2003 SP1" "5.2.3790.1830.15" "8F9E5EF3-A9A5-491B-A889-C58EFFECE8B3") +endif() +### +# Finally, look for "preferred" SDKs +### +if(_winsdk_msvc_greater_1310) # Newer than VS .NET/VS Toolkit 2003 + + + # Environment variable for SDK dir + if(EXISTS "$ENV{WindowsSDKDir}" AND (NOT "$ENV{WindowsSDKDir}" STREQUAL "")) + _winsdk_conditional_append_preferred("WindowsSDKDir environment variable" "$ENV{WindowsSDKDir}") + endif() + + if(_winsdk_msvc_less_1600) + # Per-user current Windows SDK for VS2005/2008 + get_filename_component(_sdkdir + "[HKEY_CURRENT_USER\\Software\\Microsoft\\Microsoft SDKs\\Windows;CurrentInstallFolder]" + ABSOLUTE) + _winsdk_conditional_append_preferred("Per-user current Windows SDK" "${_sdkdir}") + + # System-wide current Windows SDK for VS2005/2008 + get_filename_component(_sdkdir + "[HKEY_LOCAL_MACHINE\\SOFTWARE\\Microsoft\\Microsoft SDKs\\Windows;CurrentInstallFolder]" + ABSOLUTE) + _winsdk_conditional_append_preferred("System-wide current Windows SDK" "${_sdkdir}") + endif() +endif() + + +function(windowssdk_name_lookup _dir _outvar) + list(FIND _win_sdk_versanddirs "${_dir}" _diridx) + math(EXPR _idx "${_diridx} - 1") + if(${_idx} GREATER -1) + list(GET _win_sdk_versanddirs ${_idx} _ret) + else() + set(_ret "NOTFOUND") + endif() + set(${_outvar} "${_ret}" PARENT_SCOPE) +endfunction() + +function(windowssdk_build_lookup _dir _outvar) + list(FIND _win_sdk_buildsanddirs "${_dir}" _diridx) + math(EXPR _idx "${_diridx} - 1") + if(${_idx} GREATER -1) + list(GET _win_sdk_buildsanddirs ${_idx} _ret) + else() + set(_ret "NOTFOUND") + endif() + set(${_outvar} "${_ret}" PARENT_SCOPE) +endfunction() + +# If we found something... +if(_win_sdk_dirs) + list(GET _win_sdk_dirs 0 WINDOWSSDK_LATEST_DIR) + windowssdk_name_lookup("${WINDOWSSDK_LATEST_DIR}" + WINDOWSSDK_LATEST_NAME) + set(WINDOWSSDK_DIRS ${_win_sdk_dirs}) + + # Fallback, in case no preference found. + set(WINDOWSSDK_PREFERRED_DIR "${WINDOWSSDK_LATEST_DIR}") + set(WINDOWSSDK_PREFERRED_NAME "${WINDOWSSDK_LATEST_NAME}") + set(WINDOWSSDK_PREFERRED_FIRST_DIRS ${WINDOWSSDK_DIRS}) + set(WINDOWSSDK_FOUND_PREFERENCE OFF) +endif() + +# If we found indications of a user preference... +if(_win_sdk_preferred_sdk_dirs) + list(GET _win_sdk_preferred_sdk_dirs 0 WINDOWSSDK_PREFERRED_DIR) + windowssdk_name_lookup("${WINDOWSSDK_PREFERRED_DIR}" + WINDOWSSDK_PREFERRED_NAME) + set(WINDOWSSDK_PREFERRED_FIRST_DIRS + ${_win_sdk_preferred_sdk_dirs} + ${_win_sdk_dirs}) + list(REMOVE_DUPLICATES WINDOWSSDK_PREFERRED_FIRST_DIRS) + set(WINDOWSSDK_FOUND_PREFERENCE ON) +endif() + +include(FindPackageHandleStandardArgs) +find_package_handle_standard_args(WindowsSDK + "No compatible version of the Windows SDK or Platform SDK found." + WINDOWSSDK_DIRS) + +if(WINDOWSSDK_FOUND) + # Internal: Architecture-appropriate library directory names. + if("${CMAKE_VS_PLATFORM_NAME}" STREQUAL "ARM") + if(CMAKE_SIZEOF_VOID_P MATCHES "8") + # Only supported in Win10 SDK and up. + set(_winsdk_arch8 arm64) # what the WDK for Win8+ calls this architecture + else() + set(_winsdk_archbare /arm) # what the architecture used to be called in oldest SDKs + set(_winsdk_arch arm) # what the architecture used to be called + set(_winsdk_arch8 arm) # what the WDK for Win8+ calls this architecture + endif() + else() + if(CMAKE_SIZEOF_VOID_P MATCHES "8") + set(_winsdk_archbare /x64) # what the architecture used to be called in oldest SDKs + set(_winsdk_arch amd64) # what the architecture used to be called + set(_winsdk_arch8 x64) # what the WDK for Win8+ calls this architecture + else() + set(_winsdk_archbare ) # what the architecture used to be called in oldest SDKs + set(_winsdk_arch i386) # what the architecture used to be called + set(_winsdk_arch8 x86) # what the WDK for Win8+ calls this architecture + endif() + endif() + + function(get_windowssdk_from_component _component _var) + get_filename_component(_component "${_component}" ABSOLUTE) + file(TO_CMAKE_PATH "${_component}" _component) + foreach(_sdkdir ${WINDOWSSDK_DIRS}) + get_filename_component(_sdkdir "${_sdkdir}" ABSOLUTE) + string(LENGTH "${_sdkdir}" _sdklen) + file(RELATIVE_PATH _rel "${_sdkdir}" "${_component}") + # If we don't have any "parent directory" items... + if(NOT "${_rel}" MATCHES "[.][.]") + set(${_var} "${_sdkdir}" PARENT_SCOPE) + return() + endif() + endforeach() + # Fail. + set(${_var} "NOTFOUND" PARENT_SCOPE) + endfunction() + function(get_windowssdk_library_dirs _winsdk_dir _var) + set(_dirs) + set(_suffixes + "lib${_winsdk_archbare}" # SDKs like 7.1A + "lib/${_winsdk_arch}" # just because some SDKs have x86 dir and root dir + "lib/w2k/${_winsdk_arch}" # Win2k min requirement + "lib/wxp/${_winsdk_arch}" # WinXP min requirement + "lib/wnet/${_winsdk_arch}" # Win Server 2003 min requirement + "lib/wlh/${_winsdk_arch}" + "lib/wlh/um/${_winsdk_arch8}" # Win Vista ("Long Horn") min requirement + "lib/win7/${_winsdk_arch}" + "lib/win7/um/${_winsdk_arch8}" # Win 7 min requirement + ) + foreach(_ver + wlh # Win Vista ("Long Horn") min requirement + win7 # Win 7 min requirement + win8 # Win 8 min requirement + winv6.3 # Win 8.1 min requirement + ) + + list(APPEND _suffixes + "lib/${_ver}/${_winsdk_arch}" + "lib/${_ver}/um/${_winsdk_arch8}" + "lib/${_ver}/km/${_winsdk_arch8}" + ) + endforeach() + + # Look for WDF libraries in Win10+ SDK + foreach(_mode umdf kmdf) + file(GLOB _wdfdirs RELATIVE "${_winsdk_dir}" "${_winsdk_dir}/lib/wdf/${_mode}/${_winsdk_arch8}/*") + if(_wdfdirs) + list(APPEND _suffixes ${_wdfdirs}) + endif() + endforeach() + + # Look in each Win10+ SDK version for the components + foreach(_win10ver ${_winsdk_win10vers}) + foreach(_component um km ucrt mmos) + list(APPEND _suffixes "lib/${_win10ver}/${_component}/${_winsdk_arch8}") + endforeach() + endforeach() + + foreach(_suffix ${_suffixes}) + # Check to see if a library actually exists here. + file(GLOB _libs "${_winsdk_dir}/${_suffix}/*.lib") + if(_libs) + list(APPEND _dirs "${_winsdk_dir}/${_suffix}") + endif() + endforeach() + if("${_dirs}" STREQUAL "") + set(_dirs NOTFOUND) + else() + list(REMOVE_DUPLICATES _dirs) + endif() + set(${_var} ${_dirs} PARENT_SCOPE) + endfunction() + function(get_windowssdk_include_dirs _winsdk_dir _var) + set(_dirs) + + set(_subdirs shared um winrt km wdf mmos ucrt) + set(_suffixes Include) + + foreach(_dir ${_subdirs}) + list(APPEND _suffixes "Include/${_dir}") + endforeach() + + foreach(_ver ${_winsdk_win10vers}) + foreach(_dir ${_subdirs}) + list(APPEND _suffixes "Include/${_ver}/${_dir}") + endforeach() + endforeach() + + foreach(_suffix ${_suffixes}) + # Check to see if a header file actually exists here. + file(GLOB _headers "${_winsdk_dir}/${_suffix}/*.h") + if(_headers) + list(APPEND _dirs "${_winsdk_dir}/${_suffix}") + endif() + endforeach() + if("${_dirs}" STREQUAL "") + set(_dirs NOTFOUND) + else() + list(REMOVE_DUPLICATES _dirs) + endif() + set(${_var} ${_dirs} PARENT_SCOPE) + endfunction() + function(get_windowssdk_library_dirs_multiple _var) + set(_dirs) + foreach(_sdkdir ${ARGN}) + get_windowssdk_library_dirs("${_sdkdir}" _current_sdk_libdirs) + if(_current_sdk_libdirs) + list(APPEND _dirs ${_current_sdk_libdirs}) + endif() + endforeach() + if("${_dirs}" STREQUAL "") + set(_dirs NOTFOUND) + else() + list(REMOVE_DUPLICATES _dirs) + endif() + set(${_var} ${_dirs} PARENT_SCOPE) + endfunction() + function(get_windowssdk_include_dirs_multiple _var) + set(_dirs) + foreach(_sdkdir ${ARGN}) + get_windowssdk_include_dirs("${_sdkdir}" _current_sdk_incdirs) + if(_current_sdk_libdirs) + list(APPEND _dirs ${_current_sdk_incdirs}) + endif() + endforeach() + if("${_dirs}" STREQUAL "") + set(_dirs NOTFOUND) + else() + list(REMOVE_DUPLICATES _dirs) + endif() + set(${_var} ${_dirs} PARENT_SCOPE) + endfunction() +endif() diff --git a/stage0/src/cmake/Modules/GetGitRevisionDescription.cmake b/stage0/src/cmake/Modules/GetGitRevisionDescription.cmake index c8d27f2e8ce4..9f54191298b0 100644 --- a/stage0/src/cmake/Modules/GetGitRevisionDescription.cmake +++ b/stage0/src/cmake/Modules/GetGitRevisionDescription.cmake @@ -3,7 +3,7 @@ # These functions force a re-configure on each git commit so that you can # trust the values of the variables in your build system. # -# get_git_head_revision( [ ...]) +# get_git_head_revision( [ALLOW_LOOKING_ABOVE_CMAKE_SOURCE_DIR]) # # Returns the refspec and sha hash of the current head revision # @@ -12,26 +12,41 @@ # Returns the results of git describe on the source tree, and adjusting # the output so that it tests false if an error occurs. # +# git_describe_working_tree( [ ...]) +# +# Returns the results of git describe on the working tree (--dirty option), +# and adjusting the output so that it tests false if an error occurs. +# # git_get_exact_tag( [ ...]) # # Returns the results of git describe --exact-match on the source tree, # and adjusting the output so that it tests false if there was no exact # matching tag. # +# git_local_changes() +# +# Returns either "CLEAN" or "DIRTY" with respect to uncommitted changes. +# Uses the return code of "git diff-index --quiet HEAD --". +# Does not regard untracked files. +# # Requires CMake 2.6 or newer (uses the 'function' command) # # Original Author: -# 2009-2010 Ryan Pavlik -# http://academic.cleardefinition.com -# Iowa State University HCI Graduate Program/VRAC +# 2009-2020 Rylie Pavlik +# https://ryliepavlik.com/ +# +# Copyright 2009-2013, Iowa State University. +# Copyright 2013-2020, Rylie Pavlik +# Copyright 2013-2020, Contributors +# +# SPDX-License-Identifier: BSL-1.0 # -# Copyright Iowa State University 2009-2010. # Distributed under the Boost Software License, Version 1.0. # (See accompanying file LICENSE_1_0.txt or copy at # http://www.boost.org/LICENSE_1_0.txt) if(__get_git_revision_description) - return() + return() endif() set(__get_git_revision_description YES) @@ -39,92 +54,234 @@ set(__get_git_revision_description YES) # to find the path to this module rather than the path to a calling list file get_filename_component(_gitdescmoddir ${CMAKE_CURRENT_LIST_FILE} PATH) +# Function _git_find_closest_git_dir finds the next closest .git directory +# that is part of any directory in the path defined by _start_dir. +# The result is returned in the parent scope variable whose name is passed +# as variable _git_dir_var. If no .git directory can be found, the +# function returns an empty string via _git_dir_var. +# +# Example: Given a path C:/bla/foo/bar and assuming C:/bla/.git exists and +# neither foo nor bar contain a file/directory .git. This wil return +# C:/bla/.git +# +function(_git_find_closest_git_dir _start_dir _git_dir_var) + set(cur_dir "${_start_dir}") + set(git_dir "${_start_dir}/.git") + while(NOT EXISTS "${git_dir}") + # .git dir not found, search parent directories + set(git_previous_parent "${cur_dir}") + get_filename_component(cur_dir "${cur_dir}" DIRECTORY) + if(cur_dir STREQUAL git_previous_parent) + # We have reached the root directory, we are not in git + set(${_git_dir_var} + "" + PARENT_SCOPE) + return() + endif() + set(git_dir "${cur_dir}/.git") + endwhile() + set(${_git_dir_var} + "${git_dir}" + PARENT_SCOPE) +endfunction() + function(get_git_head_revision _refspecvar _hashvar) - set(GIT_PARENT_DIR "${CMAKE_CURRENT_SOURCE_DIR}") - set(GIT_DIR "${GIT_PARENT_DIR}/.git") - while(NOT EXISTS "${GIT_DIR}") # .git dir not found, search parent directories - set(GIT_PREVIOUS_PARENT "${GIT_PARENT_DIR}") - get_filename_component(GIT_PARENT_DIR ${GIT_PARENT_DIR} PATH) - if(GIT_PARENT_DIR STREQUAL GIT_PREVIOUS_PARENT) - # We have reached the root directory, we are not in git - set(${_refspecvar} "GITDIR-NOTFOUND" PARENT_SCOPE) - set(${_hashvar} "GITDIR-NOTFOUND" PARENT_SCOPE) - return() - endif() - set(GIT_DIR "${GIT_PARENT_DIR}/.git") - endwhile() - # check if this is a submodule - if(NOT IS_DIRECTORY ${GIT_DIR}) - file(READ ${GIT_DIR} submodule) - string(REGEX REPLACE "gitdir: (.*)\n$" "\\1" GIT_DIR_RELATIVE ${submodule}) - get_filename_component(SUBMODULE_DIR ${GIT_DIR} PATH) - get_filename_component(GIT_DIR ${SUBMODULE_DIR}/${GIT_DIR_RELATIVE} ABSOLUTE) - endif() - set(GIT_DATA "${CMAKE_CURRENT_BINARY_DIR}/CMakeFiles/git-data") - if(NOT EXISTS "${GIT_DATA}") - file(MAKE_DIRECTORY "${GIT_DATA}") - endif() - - if(NOT EXISTS "${GIT_DIR}/HEAD") - return() - endif() - set(HEAD_FILE "${GIT_DATA}/HEAD") - configure_file("${GIT_DIR}/HEAD" "${HEAD_FILE}" COPYONLY) - - configure_file("${_gitdescmoddir}/GetGitRevisionDescription.cmake.in" - "${GIT_DATA}/grabRef.cmake" - @ONLY) - include("${GIT_DATA}/grabRef.cmake") - - set(${_refspecvar} "${HEAD_REF}" PARENT_SCOPE) - set(${_hashvar} "${HEAD_HASH}" PARENT_SCOPE) + _git_find_closest_git_dir("${CMAKE_CURRENT_SOURCE_DIR}" GIT_DIR) + + if("${ARGN}" STREQUAL "ALLOW_LOOKING_ABOVE_CMAKE_SOURCE_DIR") + set(ALLOW_LOOKING_ABOVE_CMAKE_SOURCE_DIR TRUE) + else() + set(ALLOW_LOOKING_ABOVE_CMAKE_SOURCE_DIR FALSE) + endif() + if(NOT "${GIT_DIR}" STREQUAL "") + file(RELATIVE_PATH _relative_to_source_dir "${CMAKE_SOURCE_DIR}" + "${GIT_DIR}") + if("${_relative_to_source_dir}" MATCHES "[.][.]" + AND NOT ALLOW_LOOKING_ABOVE_CMAKE_SOURCE_DIR) + # We've gone above the CMake root dir. + set(GIT_DIR "") + endif() + endif() + if("${GIT_DIR}" STREQUAL "") + set(${_refspecvar} + "GITDIR-NOTFOUND" + PARENT_SCOPE) + set(${_hashvar} + "GITDIR-NOTFOUND" + PARENT_SCOPE) + return() + endif() + + # Check if the current source dir is a git submodule or a worktree. + # In both cases .git is a file instead of a directory. + # + if(NOT IS_DIRECTORY ${GIT_DIR}) + # The following git command will return a non empty string that + # points to the super project working tree if the current + # source dir is inside a git submodule. + # Otherwise the command will return an empty string. + # + execute_process( + COMMAND "${GIT_EXECUTABLE}" rev-parse + --show-superproject-working-tree + WORKING_DIRECTORY "${CMAKE_CURRENT_SOURCE_DIR}" + OUTPUT_VARIABLE out + ERROR_QUIET OUTPUT_STRIP_TRAILING_WHITESPACE) + if(NOT "${out}" STREQUAL "") + # If out is empty, GIT_DIR/CMAKE_CURRENT_SOURCE_DIR is in a submodule + file(READ ${GIT_DIR} submodule) + string(REGEX REPLACE "gitdir: (.*)$" "\\1" GIT_DIR_RELATIVE + ${submodule}) + string(STRIP ${GIT_DIR_RELATIVE} GIT_DIR_RELATIVE) + get_filename_component(SUBMODULE_DIR ${GIT_DIR} PATH) + get_filename_component(GIT_DIR ${SUBMODULE_DIR}/${GIT_DIR_RELATIVE} + ABSOLUTE) + set(HEAD_SOURCE_FILE "${GIT_DIR}/HEAD") + else() + # GIT_DIR/CMAKE_CURRENT_SOURCE_DIR is in a worktree + file(READ ${GIT_DIR} worktree_ref) + # The .git directory contains a path to the worktree information directory + # inside the parent git repo of the worktree. + # + string(REGEX REPLACE "gitdir: (.*)$" "\\1" git_worktree_dir + ${worktree_ref}) + string(STRIP ${git_worktree_dir} git_worktree_dir) + _git_find_closest_git_dir("${git_worktree_dir}" GIT_DIR) + set(HEAD_SOURCE_FILE "${git_worktree_dir}/HEAD") + endif() + else() + set(HEAD_SOURCE_FILE "${GIT_DIR}/HEAD") + endif() + set(GIT_DATA "${CMAKE_CURRENT_BINARY_DIR}/CMakeFiles/git-data") + if(NOT EXISTS "${GIT_DATA}") + file(MAKE_DIRECTORY "${GIT_DATA}") + endif() + + if(NOT EXISTS "${HEAD_SOURCE_FILE}") + return() + endif() + set(HEAD_FILE "${GIT_DATA}/HEAD") + configure_file("${HEAD_SOURCE_FILE}" "${HEAD_FILE}" COPYONLY) + + configure_file("${_gitdescmoddir}/GetGitRevisionDescription.cmake.in" + "${GIT_DATA}/grabRef.cmake" @ONLY) + include("${GIT_DATA}/grabRef.cmake") + + set(${_refspecvar} + "${HEAD_REF}" + PARENT_SCOPE) + set(${_hashvar} + "${HEAD_HASH}" + PARENT_SCOPE) endfunction() function(git_describe _var) - if(NOT GIT_FOUND) - find_package(Git QUIET) - endif() - get_git_head_revision(refspec hash) - if(NOT GIT_FOUND) - set(${_var} "GIT-NOTFOUND" PARENT_SCOPE) - return() - endif() - if(NOT hash) - set(${_var} "HEAD-HASH-NOTFOUND" PARENT_SCOPE) - return() - endif() - - # TODO sanitize - #if((${ARGN}" MATCHES "&&") OR - # (ARGN MATCHES "||") OR - # (ARGN MATCHES "\\;")) - # message("Please report the following error to the project!") - # message(FATAL_ERROR "Looks like someone's doing something nefarious with git_describe! Passed arguments ${ARGN}") - #endif() - - #message(STATUS "Arguments to execute_process: ${ARGN}") - - execute_process(COMMAND - "${GIT_EXECUTABLE}" - describe - ${hash} - ${ARGN} - WORKING_DIRECTORY - "${CMAKE_SOURCE_DIR}" - RESULT_VARIABLE - res - OUTPUT_VARIABLE - out - ERROR_QUIET - OUTPUT_STRIP_TRAILING_WHITESPACE) - if(NOT res EQUAL 0) - set(out "${out}-${res}-NOTFOUND") - endif() - - set(${_var} "${out}" PARENT_SCOPE) + if(NOT GIT_FOUND) + find_package(Git QUIET) + endif() + get_git_head_revision(refspec hash) + if(NOT GIT_FOUND) + set(${_var} + "GIT-NOTFOUND" + PARENT_SCOPE) + return() + endif() + if(NOT hash) + set(${_var} + "HEAD-HASH-NOTFOUND" + PARENT_SCOPE) + return() + endif() + + # TODO sanitize + #if((${ARGN}" MATCHES "&&") OR + # (ARGN MATCHES "||") OR + # (ARGN MATCHES "\\;")) + # message("Please report the following error to the project!") + # message(FATAL_ERROR "Looks like someone's doing something nefarious with git_describe! Passed arguments ${ARGN}") + #endif() + + #message(STATUS "Arguments to execute_process: ${ARGN}") + + execute_process( + COMMAND "${GIT_EXECUTABLE}" describe --tags --always ${hash} ${ARGN} + WORKING_DIRECTORY "${CMAKE_CURRENT_SOURCE_DIR}" + RESULT_VARIABLE res + OUTPUT_VARIABLE out + ERROR_QUIET OUTPUT_STRIP_TRAILING_WHITESPACE) + if(NOT res EQUAL 0) + set(out "${out}-${res}-NOTFOUND") + endif() + + set(${_var} + "${out}" + PARENT_SCOPE) +endfunction() + +function(git_describe_working_tree _var) + if(NOT GIT_FOUND) + find_package(Git QUIET) + endif() + if(NOT GIT_FOUND) + set(${_var} + "GIT-NOTFOUND" + PARENT_SCOPE) + return() + endif() + + execute_process( + COMMAND "${GIT_EXECUTABLE}" describe --dirty ${ARGN} + WORKING_DIRECTORY "${CMAKE_CURRENT_SOURCE_DIR}" + RESULT_VARIABLE res + OUTPUT_VARIABLE out + ERROR_QUIET OUTPUT_STRIP_TRAILING_WHITESPACE) + if(NOT res EQUAL 0) + set(out "${out}-${res}-NOTFOUND") + endif() + + set(${_var} + "${out}" + PARENT_SCOPE) endfunction() function(git_get_exact_tag _var) - git_describe(out --exact-match ${ARGN}) - set(${_var} "${out}" PARENT_SCOPE) + git_describe(out --exact-match ${ARGN}) + set(${_var} + "${out}" + PARENT_SCOPE) +endfunction() + +function(git_local_changes _var) + if(NOT GIT_FOUND) + find_package(Git QUIET) + endif() + get_git_head_revision(refspec hash) + if(NOT GIT_FOUND) + set(${_var} + "GIT-NOTFOUND" + PARENT_SCOPE) + return() + endif() + if(NOT hash) + set(${_var} + "HEAD-HASH-NOTFOUND" + PARENT_SCOPE) + return() + endif() + + execute_process( + COMMAND "${GIT_EXECUTABLE}" diff-index --quiet HEAD -- + WORKING_DIRECTORY "${CMAKE_CURRENT_SOURCE_DIR}" + RESULT_VARIABLE res + OUTPUT_VARIABLE out + ERROR_QUIET OUTPUT_STRIP_TRAILING_WHITESPACE) + if(res EQUAL 0) + set(${_var} + "CLEAN" + PARENT_SCOPE) + else() + set(${_var} + "DIRTY" + PARENT_SCOPE) + endif() endfunction() diff --git a/stage0/src/cmake/Modules/GetGitRevisionDescription.cmake.in b/stage0/src/cmake/Modules/GetGitRevisionDescription.cmake.in index 888ce13aaba3..9b8d20763759 100644 --- a/stage0/src/cmake/Modules/GetGitRevisionDescription.cmake.in +++ b/stage0/src/cmake/Modules/GetGitRevisionDescription.cmake.in @@ -1,17 +1,21 @@ -# +# # Internal file for GetGitRevisionDescription.cmake # # Requires CMake 2.6 or newer (uses the 'function' command) # # Original Author: -# 2009-2010 Ryan Pavlik -# http://academic.cleardefinition.com +# 2009-2023 Rylie Pavlik +# https://ryliepavlik.com/ # Iowa State University HCI Graduate Program/VRAC # -# Copyright Iowa State University 2009-2010. +# Copyright 2009-2012, Iowa State University +# Copyright 2011-2023, Contributors +# # Distributed under the Boost Software License, Version 1.0. # (See accompanying file LICENSE_1_0.txt or copy at # http://www.boost.org/LICENSE_1_0.txt) +# +# SPDX-License-Identifier: BSL-1.0 set(HEAD_HASH) @@ -19,20 +23,26 @@ file(READ "@HEAD_FILE@" HEAD_CONTENTS LIMIT 1024) string(STRIP "${HEAD_CONTENTS}" HEAD_CONTENTS) if(HEAD_CONTENTS MATCHES "ref") - # named branch - string(REPLACE "ref: " "" HEAD_REF "${HEAD_CONTENTS}") - if(EXISTS "@GIT_DIR@/${HEAD_REF}") - configure_file("@GIT_DIR@/${HEAD_REF}" "@GIT_DATA@/head-ref" COPYONLY) - elseif(EXISTS "@GIT_DIR@/logs/${HEAD_REF}") - configure_file("@GIT_DIR@/logs/${HEAD_REF}" "@GIT_DATA@/head-ref" COPYONLY) - set(HEAD_HASH "${HEAD_REF}") - endif() + # named branch + string(REPLACE "ref: " "" HEAD_REF "${HEAD_CONTENTS}") + if(EXISTS "@GIT_DIR@/${HEAD_REF}") + configure_file("@GIT_DIR@/${HEAD_REF}" "@GIT_DATA@/head-ref" COPYONLY) + else() + if(EXISTS "@GIT_DIR@/packed-refs") + configure_file("@GIT_DIR@/packed-refs" "@GIT_DATA@/packed-refs" + COPYONLY) + file(READ "@GIT_DATA@/packed-refs" PACKED_REFS) + if(${PACKED_REFS} MATCHES "([0-9a-z]*) ${HEAD_REF}") + set(HEAD_HASH "${CMAKE_MATCH_1}") + endif() + endif() + endif() else() - # detached HEAD - configure_file("@GIT_DIR@/HEAD" "@GIT_DATA@/head-ref" COPYONLY) + # detached HEAD + configure_file("@GIT_DIR@/HEAD" "@GIT_DATA@/head-ref" COPYONLY) endif() if(NOT HEAD_HASH) - file(READ "@GIT_DATA@/head-ref" HEAD_HASH LIMIT 1024) - string(STRIP "${HEAD_HASH}" HEAD_HASH) + file(READ "@GIT_DATA@/head-ref" HEAD_HASH LIMIT 1024) + string(STRIP "${HEAD_HASH}" HEAD_HASH) endif() diff --git a/stage0/src/cmake/Modules/README.md b/stage0/src/cmake/Modules/README.md new file mode 100644 index 000000000000..4d50b70d46d9 --- /dev/null +++ b/stage0/src/cmake/Modules/README.md @@ -0,0 +1,14 @@ +# CMake modules required for building Lean + +The files `GetGitRevisionDescription.cmake`, `GetGitRevisionDescription.cmake.in` and +`FindWindowsSDK.cmake` are part of the `cmake-modules` project by Rylie Pavlik. They +are licensed under the Boost Software License, Version 1.0. + +The modules should be updated when a new version of the Windows SDK is released. To do +so, obtain an up-to-date checkout of the `cmake-modules` project from +https://github.com/rpavlik/cmake-modules and run the following command from the root +of the `cmake-modules` repository: + +```bash +./update-modules.sh /path-to-lean4-repo/src/cmake/Modules +``` diff --git a/stage0/src/include/lean/lean.h b/stage0/src/include/lean/lean.h index c5a61269404f..a3b4a281d993 100644 --- a/stage0/src/include/lean/lean.h +++ b/stage0/src/include/lean/lean.h @@ -1847,6 +1847,140 @@ static inline uint8_t lean_usize_dec_le(size_t a1, size_t a2) { return a1 <= a2; static inline uint32_t lean_usize_to_uint32(size_t a) { return ((uint32_t)a); } static inline uint64_t lean_usize_to_uint64(size_t a) { return ((uint64_t)a); } +/* + * Note that we compile all files with -frwapv so in the following section all potential UB that + * may arise from signed overflow is forced to match 2's complement behavior. + * + * We furthermore rely on the implementation defined behavior of gcc/clang to apply reduction mod + * 2^N when casting to an integer type of size N: + * https://gcc.gnu.org/onlinedocs/gcc/Integers-implementation.html#Integers-implementation + * Unfortunately LLVM does not yet document their implementation defined behavior but it is + * most likely fine to rely on the fact that GCC and LLVM match on this: + * https://github.com/llvm/llvm-project/issues/11644 + */ + +/* Int8 */ +LEAN_EXPORT int8_t lean_int8_of_big_int(b_lean_obj_arg a); +static inline uint8_t lean_int8_of_int(b_lean_obj_arg a) { + int8_t res; + + if (lean_is_scalar(a)) { + res = (int8_t)lean_scalar_to_int64(a); + } else { + res = lean_int8_of_big_int(a); + } + + return (uint8_t)res; +} + +static inline lean_obj_res lean_int8_to_int(uint8_t a) { + int8_t arg = (int8_t)a; + return lean_int64_to_int((int64_t)arg); +} + +static inline uint8_t lean_int8_neg(uint8_t a) { + int8_t arg = (int8_t)a; + + return (uint8_t)(-arg); +} + +static inline uint8_t lean_int8_add(uint8_t a1, uint8_t a2) { + int8_t lhs = (int8_t) a1; + int8_t rhs = (int8_t) a2; + + return (uint8_t)(lhs + rhs); +} + +static inline uint8_t lean_int8_sub(uint8_t a1, uint8_t a2) { + int8_t lhs = (int8_t) a1; + int8_t rhs = (int8_t) a2; + + return (uint8_t)(lhs - rhs); +} + +static inline uint8_t lean_int8_mul(uint8_t a1, uint8_t a2) { + int8_t lhs = (int8_t) a1; + int8_t rhs = (int8_t) a2; + + return (uint8_t)(lhs * rhs); +} + +static inline uint8_t lean_int8_div(uint8_t a1, uint8_t a2) { + int8_t lhs = (int8_t) a1; + int8_t rhs = (int8_t) a2; + + return (uint8_t)(rhs == 0 ? 0 : lhs / rhs); +} + +static inline uint8_t lean_int8_mod(uint8_t a1, uint8_t a2) { + int8_t lhs = (int8_t) a1; + int8_t rhs = (int8_t) a2; + + return (uint8_t)(rhs == 0 ? 0 : lhs % rhs); +} + +static inline uint8_t lean_int8_land(uint8_t a1, uint8_t a2) { + int8_t lhs = (int8_t) a1; + int8_t rhs = (int8_t) a2; + + return (uint8_t)(lhs & rhs); +} + +static inline uint8_t lean_int8_lor(uint8_t a1, uint8_t a2) { + int8_t lhs = (int8_t) a1; + int8_t rhs = (int8_t) a2; + + return (uint8_t)(lhs | rhs); +} + +static inline uint8_t lean_int8_xor(uint8_t a1, uint8_t a2) { + int8_t lhs = (int8_t) a1; + int8_t rhs = (int8_t) a2; + + return (uint8_t)(lhs ^ rhs); +} + +static inline uint8_t lean_int8_shift_right(uint8_t a1, uint8_t a2) { + int8_t lhs = (int8_t) a1; + int8_t rhs = (int8_t) a2; + + return (uint8_t)(lhs >> (rhs % 8)); +} + +static inline uint8_t lean_int8_shift_left(uint8_t a1, uint8_t a2) { + int8_t lhs = (int8_t) a1; + int8_t rhs = (int8_t) a2; + + return (uint8_t)(lhs << (rhs % 8)); +} + +static inline uint8_t lean_int8_complement(uint8_t a) { + int8_t arg = (int8_t)a; + + return (uint8_t)(~arg); +} + +static inline uint8_t lean_int8_dec_eq(uint8_t a1, uint8_t a2) { + int8_t lhs = (int8_t) a1; + int8_t rhs = (int8_t) a2; + + return lhs == rhs; +} + +static inline uint8_t lean_int8_dec_lt(uint8_t a1, uint8_t a2) { + int8_t lhs = (int8_t) a1; + int8_t rhs = (int8_t) a2; + + return lhs < rhs; +} + +static inline uint8_t lean_int8_dec_le(uint8_t a1, uint8_t a2) { + int8_t lhs = (int8_t) a1; + int8_t rhs = (int8_t) a2; + + return lhs <= rhs; +} + /* Float */ LEAN_EXPORT lean_obj_res lean_float_to_string(double a); diff --git a/stage0/src/kernel/declaration.cpp b/stage0/src/kernel/declaration.cpp index 489a134c1258..492d3942c88b 100644 --- a/stage0/src/kernel/declaration.cpp +++ b/stage0/src/kernel/declaration.cpp @@ -126,7 +126,6 @@ constructor_val::constructor_val(name const & n, names const & lparams, expr con object_ref(lean_mk_constructor_val(n.to_obj_arg(), lparams.to_obj_arg(), type.to_obj_arg(), induct.to_obj_arg(), nat(cidx).to_obj_arg(), nat(nparams).to_obj_arg(), nat(nfields).to_obj_arg(), is_unsafe)) { } - bool constructor_val::is_unsafe() const { return lean_constructor_val_is_unsafe(to_obj_arg()); } extern "C" object * lean_mk_recursor_val(object * n, object * lparams, object * type, object * all, @@ -143,6 +142,18 @@ recursor_val::recursor_val(name const & n, names const & lparams, expr const & t nat(nminors).to_obj_arg(), rules.to_obj_arg(), k, is_unsafe)) { } +name const & recursor_val::get_major_induct() const { + unsigned int n = get_major_idx(); + expr const * t = &(to_constant_val().get_type()); + for (unsigned int i = 0; i < n; i++) { + t = &(binding_body(*t)); + } + t = &(binding_domain(*t)); + t = &(get_app_fn(*t)); + return const_name(*t); +} + + bool recursor_val::is_k() const { return lean_recursor_k(to_obj_arg()); } bool recursor_val::is_unsafe() const { return lean_recursor_is_unsafe(to_obj_arg()); } diff --git a/stage0/src/kernel/declaration.h b/stage0/src/kernel/declaration.h index 9b636ae0a8f6..398d4e1f8967 100644 --- a/stage0/src/kernel/declaration.h +++ b/stage0/src/kernel/declaration.h @@ -370,7 +370,7 @@ class recursor_val : public object_ref { recursor_val & operator=(recursor_val && other) { object_ref::operator=(std::move(other)); return *this; } constant_val const & to_constant_val() const { return static_cast(cnstr_get_ref(*this, 0)); } name const & get_name() const { return to_constant_val().get_name(); } - name const & get_induct() const { return get_name().get_prefix(); } + name const & get_major_induct() const; names const & get_all() const { return static_cast(cnstr_get_ref(*this, 1)); } unsigned get_nparams() const { return static_cast(cnstr_get_ref(*this, 2)).get_small_value(); } unsigned get_nindices() const { return static_cast(cnstr_get_ref(*this, 3)).get_small_value(); } diff --git a/stage0/src/kernel/expr.cpp b/stage0/src/kernel/expr.cpp index 983764623727..957809c2e3aa 100644 --- a/stage0/src/kernel/expr.cpp +++ b/stage0/src/kernel/expr.cpp @@ -79,21 +79,22 @@ extern "C" object * lean_lit_type(obj_arg e); expr lit_type(literal const & lit) { return expr(lean_lit_type(lit.to_obj_arg())); } extern "C" uint64_t lean_expr_hash(obj_arg e); -unsigned hash(expr const & e) { - object * o = e.raw(); - unsigned r = static_cast(lean_ctor_get_uint64(o, lean_ctor_num_objs(o)*sizeof(object*))); - lean_assert(r == lean_expr_hash(e.to_obj_arg())); - return r; +unsigned hash_core(expr const & e) { + return lean_expr_hash(e.to_obj_arg()); } extern "C" uint8 lean_expr_has_fvar(obj_arg e); -bool has_fvar(expr const & e) { return lean_expr_has_fvar(e.to_obj_arg()); } +bool has_fvar_core(expr const & e) { + return lean_expr_has_fvar(e.to_obj_arg()); +} extern "C" uint8 lean_expr_has_expr_mvar(obj_arg e); -bool has_expr_mvar(expr const & e) { return lean_expr_has_expr_mvar(e.to_obj_arg()); } +bool has_expr_mvar_core(expr const & e) { + return lean_expr_has_expr_mvar(e.to_obj_arg()); +} extern "C" uint8 lean_expr_has_level_mvar(obj_arg e); -bool has_univ_mvar(expr const & e) { return lean_expr_has_level_mvar(e.to_obj_arg()); } +bool has_univ_mvar_core(expr const & e) { return lean_expr_has_level_mvar(e.to_obj_arg()); } extern "C" uint8 lean_expr_has_level_param(obj_arg e); bool has_univ_param(expr const & e) { return lean_expr_has_level_param(e.to_obj_arg()); } diff --git a/stage0/src/kernel/expr.h b/stage0/src/kernel/expr.h index d1771e73a366..c110ebd26c32 100644 --- a/stage0/src/kernel/expr.h +++ b/stage0/src/kernel/expr.h @@ -123,11 +123,37 @@ inline bool is_eqp(optional const & a, optional const & b) { return static_cast(a) == static_cast(b) && (!a || is_eqp(*a, *b)); } -unsigned hash(expr const & e); -bool has_expr_mvar(expr const & e); -bool has_univ_mvar(expr const & e); +inline uint64_t get_data(expr const & e) { + return lean_ctor_get_uint64(e.raw(), lean_ctor_num_objs(e.raw())*sizeof(object*)); +} +/* This is the implementation in Lean */ +unsigned hash_core(expr const & e); +inline unsigned hash(expr const & e) { + unsigned r = static_cast(get_data(e)); + lean_assert(r == hash_core(e)); + return r; +} +/* This is the implementation in Lean */ +bool has_expr_mvar_core(expr const & e); +inline bool has_expr_mvar(expr const & e) { + bool r = ((get_data(e) >> 41) & 1) == 1; + lean_assert(r == has_expr_mvar_core(e)); // ensure the C++ implementation matches the Lean one. + return r; +} +bool has_univ_mvar_core(expr const & e); +inline bool has_univ_mvar(expr const & e) { + bool r = ((get_data(e) >> 42) & 1) == 1; + lean_assert(r == has_univ_mvar_core(e)); // ensure the C++ implementation matches the Lean one. + return r; +} inline bool has_mvar(expr const & e) { return has_expr_mvar(e) || has_univ_mvar(e); } -bool has_fvar(expr const & e); +/* This is the implementation in Lean */ +bool has_fvar_core(expr const & e); +inline bool has_fvar(expr const & e) { + bool r = ((get_data(e) >> 40) & 1) == 1; + lean_assert(r == has_fvar_core(e)); // ensure the C++ implementation matches the Lean one. + return r; +} bool has_univ_param(expr const & e); unsigned get_loose_bvar_range(expr const & e); diff --git a/stage0/src/kernel/inductive.h b/stage0/src/kernel/inductive.h index dd6b2671b2bf..a7b2864624ac 100644 --- a/stage0/src/kernel/inductive.h +++ b/stage0/src/kernel/inductive.h @@ -33,7 +33,7 @@ inline expr to_cnstr_when_K(environment const & env, recursor_val const & rval, lean_assert(rval.is_k()); expr app_type = whnf(infer_type(e)); expr const & app_type_I = get_app_fn(app_type); - if (!is_constant(app_type_I) || const_name(app_type_I) != rval.get_induct()) return e; // type incorrect + if (!is_constant(app_type_I) || const_name(app_type_I) != rval.get_major_induct()) return e; // type incorrect if (has_expr_mvar(app_type)) { buffer app_type_args; get_app_args(app_type, app_type_args); @@ -94,7 +94,7 @@ inline optional inductive_reduce_rec(environment const & env, expr const & else if (is_string_lit(major)) major = string_lit_to_constructor(major); else - major = to_cnstr_when_structure(env, rec_val.get_induct(), major, whnf, infer_type); + major = to_cnstr_when_structure(env, rec_val.get_major_induct(), major, whnf, infer_type); optional rule = get_rec_rule_for(rec_val, major); if (!rule) return none_expr(); buffer major_args; diff --git a/stage0/src/kernel/replace_fn.cpp b/stage0/src/kernel/replace_fn.cpp index 0a2b1030d12b..f97ef05cc630 100644 --- a/stage0/src/kernel/replace_fn.cpp +++ b/stage0/src/kernel/replace_fn.cpp @@ -12,6 +12,23 @@ Author: Leonardo de Moura namespace lean { +/* Like `is_exclusive`, but also consider unique MT references as unshared, which ensures we get + * similar performance on the cmdline and server (more precisely, for either option value of + * `internal.cmdlineSnapshots`). Note that as `e` is merely *borrowed* (e.g. from the mctx in + * the case of `instantiate_mvars` where the performance issue resolved here manifested, #5614), + * it is in fact possible that another thread could simultaneously add a new direct reference to + * `e`, so it is not definitely unshared in all cases if the below check is true. + * + * However, as we use this predicate merely as a conservative heuristic for detecting + * expressions that are unshared *within the expression tree* at hand, the approximation is + * still correct in this case. Furthermore, as we only use it for deciding when to cache + * results, it ultimately does not affect the correctness of the overall procedure in any case. + * This should however be kept in mind if we start using `is_likely_unshared` in other contexts. + */ +static bool is_likely_unshared(expr const & e) { + return e.raw()->m_rc == 1 || e.raw()->m_rc == -1; +} + class replace_rec_fn { struct key_hasher { std::size_t operator()(std::pair const & p) const { @@ -30,7 +47,7 @@ class replace_rec_fn { expr apply(expr const & e, unsigned offset) { bool shared = false; - if (m_use_cache && is_shared(e)) { + if (m_use_cache && !is_likely_unshared(e)) { auto it = m_cache.find(mk_pair(e.raw(), offset)); if (it != m_cache.end()) return it->second; diff --git a/stage0/src/runtime/hash.h b/stage0/src/runtime/hash.h index 4fcb70b8a682..105ec6ca67d3 100644 --- a/stage0/src/runtime/hash.h +++ b/stage0/src/runtime/hash.h @@ -6,7 +6,7 @@ Author: Leonardo de Moura */ #pragma once #include "runtime/debug.h" -#include "runtime/int64.h" +#include "runtime/int.h" namespace lean { diff --git a/stage0/src/runtime/int.h b/stage0/src/runtime/int.h new file mode 100644 index 000000000000..1163570244eb --- /dev/null +++ b/stage0/src/runtime/int.h @@ -0,0 +1,33 @@ +/* +Copyright (c) 2013 Microsoft Corporation. All rights reserved. +Released under Apache 2.0 license as described in the file LICENSE. + +Author: Leonardo de Moura +*/ +#include +#include +namespace lean { + +typedef int8_t int8; +typedef uint8_t uint8; +static_assert(sizeof(int8) == 1, "unexpected int8 size"); // NOLINT +static_assert(sizeof(uint8) == 1, "unexpected uint8 size"); // NOLINT + // +typedef int16_t int16; +typedef uint16_t uint16; +static_assert(sizeof(int16) == 2, "unexpected int16 size"); // NOLINT +static_assert(sizeof(uint16) == 2, "unexpected uint16 size"); // NOLINT + // +typedef int32_t int32; +typedef uint32_t uint32; +static_assert(sizeof(int32) == 4, "unexpected int32 size"); // NOLINT +static_assert(sizeof(uint32) == 4, "unexpected uint32 size"); // NOLINT + +typedef int64_t int64; +typedef uint64_t uint64; +static_assert(sizeof(int64) == 8, "unexpected int64 size"); // NOLINT +static_assert(sizeof(uint64) == 8, "unexpected uint64 size"); // NOLINT + // +typedef size_t usize; + +} diff --git a/stage0/src/runtime/int64.h b/stage0/src/runtime/int64.h deleted file mode 100644 index 47f6ef33dcbd..000000000000 --- a/stage0/src/runtime/int64.h +++ /dev/null @@ -1,13 +0,0 @@ -/* -Copyright (c) 2013 Microsoft Corporation. All rights reserved. -Released under Apache 2.0 license as described in the file LICENSE. - -Author: Leonardo de Moura -*/ -#include -namespace lean { -typedef int64_t int64; -typedef uint64_t uint64; -static_assert(sizeof(int64) == 8, "unexpected int64 size"); // NOLINT -static_assert(sizeof(uint64) == 8, "unexpected uint64 size"); // NOLINT -} diff --git a/stage0/src/runtime/mpz.cpp b/stage0/src/runtime/mpz.cpp index 8dc4a71c7d3c..b1d1af9e0d4e 100644 --- a/stage0/src/runtime/mpz.cpp +++ b/stage0/src/runtime/mpz.cpp @@ -239,22 +239,22 @@ void div2k(mpz & a, mpz const & b, unsigned k) { mpz_tdiv_q_2exp(a.m_val, b.m_val, k); } -unsigned mpz::mod8() const { +uint8 mpz::mod8() const { mpz a; mpz_tdiv_r_2exp(a.m_val, m_val, 8); - return a.get_unsigned_int(); + return static_cast(a.get_unsigned_int()); } -unsigned mpz::mod16() const { +uint16 mpz::mod16() const { mpz a; mpz_tdiv_r_2exp(a.m_val, m_val, 16); - return a.get_unsigned_int(); + return static_cast(a.get_unsigned_int()); } -unsigned mpz::mod32() const { +uint32 mpz::mod32() const { mpz a; mpz_tdiv_r_2exp(a.m_val, m_val, 32); - return a.get_unsigned_int(); + return static_cast(a.get_unsigned_int()); } uint64 mpz::mod64() const { @@ -267,6 +267,12 @@ uint64 mpz::mod64() const { return (static_cast(h.get_unsigned_int()) << 32) + static_cast(l.get_unsigned_int()); } +int8 mpz::smod8() const { + mpz a; + mpz_tdiv_r_2exp(a.m_val, m_val, 8); + return static_cast(a.get_int()); +} + void power(mpz & a, mpz const & b, unsigned k) { mpz_pow_ui(a.m_val, b.m_val, k); } @@ -945,16 +951,16 @@ void div2k(mpz & a, mpz const & b, unsigned k) { a.set(new_sz, ds.begin()); } -unsigned mpz::mod8() const { - return m_digits[0] & 0xFFu; +uint8 mpz::mod8() const { + return static_cast(m_digits[0] & 0xFFu); } -unsigned mpz::mod16() const { - return m_digits[0] & 0xFFFFu; +uint16 mpz::mod16() const { + return static_cast(m_digits[0] & 0xFFFFu); } -unsigned mpz::mod32() const { - return m_digits[0]; +uint32 mpz::mod32() const { + return static_cast(m_digits[0]); } uint64 mpz::mod64() const { @@ -964,6 +970,14 @@ uint64 mpz::mod64() const { return m_digits[0] + (static_cast(m_digits[1]) << 8*sizeof(mpn_digit)); } +int8 mpz::smod8() const { + int8_t val = mod8(); + if (m_sign) { + val = -val; + } + return val; +} + void power(mpz & a, mpz const & b, unsigned k) { a = b; a.pow(k); diff --git a/stage0/src/runtime/mpz.h b/stage0/src/runtime/mpz.h index 68127c4606fd..82f1a283dcb4 100644 --- a/stage0/src/runtime/mpz.h +++ b/stage0/src/runtime/mpz.h @@ -15,7 +15,7 @@ Author: Leonardo de Moura #include #include #include -#include "runtime/int64.h" +#include "runtime/int.h" #include "runtime/debug.h" namespace lean { @@ -266,11 +266,13 @@ class LEAN_EXPORT mpz { // a <- b / 2^k friend void div2k(mpz & a, mpz const & b, unsigned k); - unsigned mod8() const; - unsigned mod16() const; - unsigned mod32() const; + uint8 mod8() const; + uint16 mod16() const; + uint32 mod32() const; uint64 mod64() const; + int8 smod8() const; + /** \brief Return the position of the most significant bit. Return 0 if the number is negative diff --git a/stage0/src/runtime/object.cpp b/stage0/src/runtime/object.cpp index eb6461f7cf8f..8d0f59c47914 100644 --- a/stage0/src/runtime/object.cpp +++ b/stage0/src/runtime/object.cpp @@ -1536,11 +1536,11 @@ extern "C" LEAN_EXPORT bool lean_int_big_nonneg(object * a) { // UInt extern "C" LEAN_EXPORT uint8 lean_uint8_of_big_nat(b_obj_arg a) { - return static_cast(mpz_value(a).mod8()); + return mpz_value(a).mod8(); } extern "C" LEAN_EXPORT uint16 lean_uint16_of_big_nat(b_obj_arg a) { - return static_cast(mpz_value(a).mod16()); + return mpz_value(a).mod16(); } extern "C" LEAN_EXPORT uint32 lean_uint32_of_big_nat(b_obj_arg a) { @@ -1574,6 +1574,13 @@ extern "C" LEAN_EXPORT usize lean_usize_big_modn(usize a1, b_lean_obj_arg) { return a1; } +// ======================================= +// IntX + +extern "C" LEAN_EXPORT int8 lean_int8_of_big_int(b_obj_arg a) { + return mpz_value(a).smod8(); +} + // ======================================= // Float diff --git a/stage0/src/runtime/object.h b/stage0/src/runtime/object.h index b5e5a6375817..24ebe298a595 100644 --- a/stage0/src/runtime/object.h +++ b/stage0/src/runtime/object.h @@ -10,11 +10,6 @@ Author: Leonardo de Moura #include "runtime/mpz.h" namespace lean { -typedef uint8_t uint8; -typedef uint16_t uint16; -typedef uint32_t uint32; -typedef uint64_t uint64; -typedef size_t usize; typedef lean_object object; typedef object * obj_arg; diff --git a/stage0/src/util/message_definitions.h b/stage0/src/util/message_definitions.h index 94aa8cf65990..53426634ffa3 100644 --- a/stage0/src/util/message_definitions.h +++ b/stage0/src/util/message_definitions.h @@ -7,7 +7,7 @@ Author: Gabriel Ebner #pragma once #include #include -#include "runtime/int64.h" +#include "runtime/int.h" #include "util/name.h" namespace lean { diff --git a/stage0/stdlib/Init.c b/stage0/stdlib/Init.c index 09ae651f8920..3b6237764369 100644 --- a/stage0/stdlib/Init.c +++ b/stage0/stdlib/Init.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Init -// Imports: Init.Prelude Init.Notation Init.Tactics Init.TacticsExtra Init.ByCases Init.RCases Init.Core Init.Control Init.Data.Basic Init.WF Init.WFTactics Init.Data Init.System Init.Util Init.Dynamic Init.ShareCommon Init.MetaTypes Init.Meta Init.NotationExtra Init.SimpLemmas Init.PropLemmas Init.Hints Init.Conv Init.Guard Init.Simproc Init.SizeOfLemmas Init.BinderPredicates Init.Ext Init.Omega Init.MacroTrace Init.Grind +// Imports: Init.Prelude Init.Notation Init.Tactics Init.TacticsExtra Init.ByCases Init.RCases Init.Core Init.Control Init.Data.Basic Init.WF Init.WFTactics Init.Data Init.System Init.Util Init.Dynamic Init.ShareCommon Init.MetaTypes Init.Meta Init.NotationExtra Init.SimpLemmas Init.PropLemmas Init.Hints Init.Conv Init.Guard Init.Simproc Init.SizeOfLemmas Init.BinderPredicates Init.Ext Init.Omega Init.MacroTrace Init.Grind Init.While #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -44,6 +44,7 @@ lean_object* initialize_Init_Ext(uint8_t builtin, lean_object*); lean_object* initialize_Init_Omega(uint8_t builtin, lean_object*); lean_object* initialize_Init_MacroTrace(uint8_t builtin, lean_object*); lean_object* initialize_Init_Grind(uint8_t builtin, lean_object*); +lean_object* initialize_Init_While(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Init(uint8_t builtin, lean_object* w) { lean_object * res; @@ -142,6 +143,9 @@ lean_dec_ref(res); res = initialize_Init_Grind(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +res = initialize_Init_While(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Init/Control/Basic.c b/stage0/stdlib/Init/Control/Basic.c index f4731fd661fb..d2cc91c39a6b 100644 --- a/stage0/stdlib/Init/Control/Basic.c +++ b/stage0/stdlib/Init/Control/Basic.c @@ -41,6 +41,7 @@ LEAN_EXPORT lean_object* l_Bind_kleisliLeft(lean_object*, lean_object*, lean_obj LEAN_EXPORT lean_object* l___aux__Init__Control__Basic______unexpand__andM__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_instToBoolBool___boxed(lean_object*); LEAN_EXPORT lean_object* l_bool___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_instForInOfForIn_x27(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__Control__Basic______macroRules__term___x3e_x3d_x3e____1___closed__2; lean_object* l_Lean_replaceRef(lean_object*, lean_object*); static lean_object* l___aux__Init__Control__Basic______macroRules__term___x3c_x26_x3e____1___closed__3; @@ -53,6 +54,7 @@ static lean_object* l___aux__Init__Control__Basic______macroRules__term___x3c_x2 static lean_object* l___aux__Init__Control__Basic______macroRules__term___x3c_x7c_x7c_x3e____1___closed__2; LEAN_EXPORT lean_object* l_term___x3c_x26_x26_x3e__; uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_instForInOfForIn_x27___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_orM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___aux__Init__Control__Basic______unexpand__Bind__kleisliRight__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_andM___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); @@ -66,6 +68,7 @@ static lean_object* l___aux__Init__Control__Basic______macroRules__term___x3c_x2 static lean_object* l_term___x3d_x3c_x3c_____closed__5; static lean_object* l_term___x3c_x26_x3e_____closed__8; LEAN_EXPORT lean_object* l_orM___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_instForInOfForIn_x27___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__Control__Basic______macroRules__term___x3c_x7c_x7c_x3e____1___closed__3; static lean_object* l_term___x3c_x26_x26_x3e_____closed__3; LEAN_EXPORT lean_object* l_instMonadControlTOfMonadControl___rarg(lean_object*, lean_object*); @@ -167,6 +170,7 @@ LEAN_EXPORT lean_object* l_control___rarg(lean_object*, lean_object*, lean_objec LEAN_EXPORT lean_object* l_bool___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_term___x3c_x3d_x3c_____closed__6; LEAN_EXPORT lean_object* l_guard___rarg___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_instForInOfForIn_x27___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__Control__Basic______macroRules__term___x3c_x7c_x7c_x3e____1___closed__5; LEAN_EXPORT lean_object* l___aux__Init__Control__Basic______macroRules__term___x3c_x7c_x7c_x3e____1(lean_object*, lean_object*, lean_object*); static lean_object* l_term___x3c_x7c_x7c_x3e_____closed__3; @@ -195,6 +199,41 @@ LEAN_EXPORT lean_object* l_optional(lean_object*); LEAN_EXPORT lean_object* l_term___x3c_x7c_x7c_x3e__; static lean_object* l___aux__Init__Control__Basic______macroRules__term___x3d_x3c_x3c____1___closed__3; static lean_object* l_term___x3c_x26_x3e_____closed__4; +LEAN_EXPORT lean_object* l_instForInOfForIn_x27___rarg___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 = lean_apply_2(x_1, x_2, x_4); +return x_5; +} +} +LEAN_EXPORT lean_object* l_instForInOfForIn_x27___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; +x_7 = lean_alloc_closure((void*)(l_instForInOfForIn_x27___rarg___lambda__1), 4, 1); +lean_closure_set(x_7, 0, x_6); +x_8 = lean_apply_5(x_1, lean_box(0), x_3, x_4, x_5, x_7); +return x_8; +} +} +LEAN_EXPORT lean_object* l_instForInOfForIn_x27(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_instForInOfForIn_x27___rarg), 6, 0); +return x_5; +} +} +LEAN_EXPORT lean_object* l_instForInOfForIn_x27___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_instForInOfForIn_x27(x_1, x_2, x_3, x_4); +lean_dec(x_4); +return x_5; +} +} LEAN_EXPORT lean_object* l_Functor_mapRev___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { diff --git a/stage0/stdlib/Init/Control/StateRef.c b/stage0/stdlib/Init/Control/StateRef.c index 2ba3be75fcf0..e2bea9c205cd 100644 --- a/stage0/stdlib/Init/Control/StateRef.c +++ b/stage0/stdlib/Init/Control/StateRef.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Init.Control.StateRef -// Imports: Init.System.IO Init.Control.State +// Imports: Init.System.ST #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -506,17 +506,13 @@ x_4 = lean_alloc_closure((void*)(l_instMonadFinallyStateRefT_x27___rarg), 1, 0); return x_4; } } -lean_object* initialize_Init_System_IO(uint8_t builtin, lean_object*); -lean_object* initialize_Init_Control_State(uint8_t builtin, lean_object*); +lean_object* initialize_Init_System_ST(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Init_Control_StateRef(uint8_t builtin, lean_object* w) { lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init_System_IO(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -res = initialize_Init_Control_State(builtin, lean_io_mk_world()); +res = initialize_Init_System_ST(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); l_StateRefT_x27_instMonadLift___closed__1 = _init_l_StateRefT_x27_instMonadLift___closed__1(); diff --git a/stage0/stdlib/Init/Data.c b/stage0/stdlib/Init/Data.c index ca08a95ee6fc..9dd257169eee 100644 --- a/stage0/stdlib/Init/Data.c +++ b/stage0/stdlib/Init/Data.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Init.Data -// Imports: Init.Data.Basic Init.Data.Nat Init.Data.Bool Init.Data.BitVec Init.Data.Cast Init.Data.Char Init.Data.String Init.Data.List Init.Data.Int Init.Data.Array Init.Data.Array.Subarray.Split Init.Data.ByteArray Init.Data.FloatArray Init.Data.Fin Init.Data.UInt Init.Data.Float Init.Data.Option Init.Data.Ord Init.Data.Random Init.Data.ToString Init.Data.Range Init.Data.Hashable Init.Data.OfScientific Init.Data.Format Init.Data.Stream Init.Data.Prod Init.Data.AC Init.Data.Queue Init.Data.Channel Init.Data.Sum Init.Data.BEq Init.Data.Subtype Init.Data.ULift Init.Data.PLift Init.Data.Zero Init.Data.NeZero Init.Data.Function +// Imports: Init.Data.Basic Init.Data.Nat Init.Data.Bool Init.Data.BitVec Init.Data.Cast Init.Data.Char Init.Data.String Init.Data.List Init.Data.Int Init.Data.Array Init.Data.Array.Subarray.Split Init.Data.ByteArray Init.Data.FloatArray Init.Data.Fin Init.Data.UInt Init.Data.SInt Init.Data.Float Init.Data.Option Init.Data.Ord Init.Data.Random Init.Data.ToString Init.Data.Range Init.Data.Hashable Init.Data.OfScientific Init.Data.Format Init.Data.Stream Init.Data.Prod Init.Data.AC Init.Data.Queue Init.Data.Channel Init.Data.Sum Init.Data.BEq Init.Data.Subtype Init.Data.ULift Init.Data.PLift Init.Data.Zero Init.Data.NeZero Init.Data.Function #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -28,6 +28,7 @@ lean_object* initialize_Init_Data_ByteArray(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_FloatArray(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_Fin(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_UInt(uint8_t builtin, lean_object*); +lean_object* initialize_Init_Data_SInt(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_Float(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_Option(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_Ord(uint8_t builtin, lean_object*); @@ -100,6 +101,9 @@ lean_dec_ref(res); res = initialize_Init_Data_UInt(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +res = initialize_Init_Data_SInt(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); res = initialize_Init_Data_Float(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Init/Data/Array.c b/stage0/stdlib/Init/Data/Array.c index a906ba7df467..2dc8f1febdc8 100644 --- a/stage0/stdlib/Init/Data/Array.c +++ b/stage0/stdlib/Init/Data/Array.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Init.Data.Array -// Imports: Init.Data.Array.Basic Init.Data.Array.QSort Init.Data.Array.BinSearch Init.Data.Array.InsertionSort Init.Data.Array.DecidableEq Init.Data.Array.Mem Init.Data.Array.Attach Init.Data.Array.BasicAux Init.Data.Array.Lemmas Init.Data.Array.TakeDrop Init.Data.Array.Bootstrap Init.Data.Array.GetLit +// Imports: Init.Data.Array.Basic Init.Data.Array.QSort Init.Data.Array.BinSearch Init.Data.Array.InsertionSort Init.Data.Array.DecidableEq Init.Data.Array.Mem Init.Data.Array.Attach Init.Data.Array.BasicAux Init.Data.Array.Lemmas Init.Data.Array.TakeDrop Init.Data.Array.Bootstrap Init.Data.Array.GetLit Init.Data.Array.MapIdx #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -25,6 +25,7 @@ lean_object* initialize_Init_Data_Array_Lemmas(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_Array_TakeDrop(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_Array_Bootstrap(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_Array_GetLit(uint8_t builtin, lean_object*); +lean_object* initialize_Init_Data_Array_MapIdx(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Init_Data_Array(uint8_t builtin, lean_object* w) { lean_object * res; @@ -66,6 +67,9 @@ lean_dec_ref(res); res = initialize_Init_Data_Array_GetLit(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +res = initialize_Init_Data_Array_MapIdx(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Init/Data/Array/Basic.c b/stage0/stdlib/Init/Data/Array/Basic.c index ef545f538a83..7fbe3eab2833 100644 --- a/stage0/stdlib/Init/Data/Array/Basic.c +++ b/stage0/stdlib/Init/Data/Array/Basic.c @@ -18,11 +18,15 @@ LEAN_EXPORT lean_object* l_Array_filterM___rarg(lean_object*, lean_object*, lean LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at_Array_findRevM_x3f___spec__1___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_concatMapM(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_takeWhile(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapIdxM___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__5; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_reduceOption___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Array_isPrefixOf(lean_object*); +LEAN_EXPORT lean_object* l_Array_take___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Nat_foldTR_loop___at_Array_range___spec__1___at_Array_range___spec__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_foldl___spec__1___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_term_x23_x5b___x2c_x5d___closed__15; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_zipWithIndex___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findRev_x3f___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrM_fold___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_instAppend(lean_object*); @@ -32,12 +36,14 @@ LEAN_EXPORT lean_object* l_Array_uget___boxed(lean_object*, lean_object*, lean_o LEAN_EXPORT uint8_t l_Array_isEqvAux___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Array_swapAt_x21___spec__1(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_allDiffAux(lean_object*); +LEAN_EXPORT lean_object* l_Array_instForIn_x27InferInstanceMembership(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_toListAppend___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Array_contains___spec__1(lean_object*); static lean_object* l_Array_instRepr___rarg___closed__5; static lean_object* l_term_x23_x5b___x2c_x5d___closed__14; LEAN_EXPORT lean_object* l_Array_foldlM_loop___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_data(lean_object*); LEAN_EXPORT lean_object* l_Array_findSomeM_x3f___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_eraseReps___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_insertAt_loop___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -47,8 +53,8 @@ static lean_object* l___aux__Init__Data__Array__Basic______macroRules__term_x23_ LEAN_EXPORT lean_object* l_Array_findSome_x21___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_modifyMUnsafe___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatten___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapFinIdx___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Array_find_x3f___spec__1(lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Array_findM_x3f___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_ofFn_go___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_loop___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -64,6 +70,7 @@ static lean_object* l___aux__Init__Data__Array__Basic______macroRules__term_x23_ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_getEvenElems___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_forRevM___spec__2___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_term_x23_x5b___x2c_x5d___closed__7; +LEAN_EXPORT lean_object* l_Array_forIn_x27_loop(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_erase___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findSomeRev_x3f___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_eraseReps___rarg(lean_object*, lean_object*); @@ -89,6 +96,7 @@ LEAN_EXPORT lean_object* l_Array_allDiff___rarg___boxed(lean_object*, lean_objec lean_object* lean_array_push(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_toListAppend___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_flatten___rarg___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Array_flatMap___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_filterMap___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -110,6 +118,7 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Array_findSomeM_x3f___spe LEAN_EXPORT lean_object* l_Array_instGetElemUSizeLtNatToNatSize(lean_object*); LEAN_EXPORT lean_object* l_panic___at_Array_swapAt_x21___spec__1___rarg(lean_object*, lean_object*, lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_reduceOption___spec__2___rarg(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_forM___spec__1___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_getIdx_x3f(lean_object*); @@ -122,7 +131,8 @@ LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Array_contains___spec__1___rarg( static lean_object* l_Array_instRepr___rarg___closed__8; LEAN_EXPORT lean_object* l_Array_findIdx_x3f_loop___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_foldr___spec__2___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Nat_foldTR_loop___at_Array_range___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyM_loop___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at_Array_findRev_x3f___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -131,6 +141,7 @@ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_toListAppend___spe LEAN_EXPORT lean_object* l_Array_unzip(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Array_findSomeM_x3f___spec__1___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_filterMapM___at_Array_reduceOption___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_loop___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Array_findIdxM_x3f___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Array_findIdxM_x3f___spec__1___rarg___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -150,8 +161,10 @@ LEAN_EXPORT lean_object* l_Array_back(lean_object*); LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at_Array_findSomeRev_x3f___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mkArray___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_swapAt(lean_object*); +LEAN_EXPORT lean_object* l_Array_instForIn_x27InferInstanceMembership___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_zipWithAux(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyM_loop(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_filterMapM___at_Array_reduceOption___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Array_findSomeM_x3f___rarg___lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_any___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Array_findIdxM_x3f___spec__1(lean_object*, lean_object*); @@ -169,9 +182,11 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec_ static lean_object* l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__18; LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_find_x3f___rarg___closed__2; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_reduceOption___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forRevM___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_split___spec__1___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__1; +LEAN_EXPORT lean_object* l_Array_instMembership(lean_object*); LEAN_EXPORT lean_object* l_Array_concatMap___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forM___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_term_x23_x5b___x2c_x5d___closed__10; @@ -182,26 +197,31 @@ LEAN_EXPORT lean_object* l_Array_isEqv(lean_object*); LEAN_EXPORT lean_object* l_Array_mapIdx(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_forM___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_unzip___rarg___closed__1; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrM_fold(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_modify(lean_object*); +LEAN_EXPORT lean_object* l_Array_take___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_loop___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_split___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlM_loop(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_instHAppendList(lean_object*); +LEAN_EXPORT lean_object* l_Array_take(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlM_loop___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_instEmptyCollection(lean_object*); +LEAN_EXPORT lean_object* l_Array_take_loop(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_foldl___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_swapAt_x21___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapIdx___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_isEmpty(lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapM_map___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Array_zipWithIndex___spec__1(lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27_loop___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_singleton(lean_object*); LEAN_EXPORT lean_object* l_Array_findSomeM_x3f___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_flatMap(lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Array_map(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findRev_x3f___rarg___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_concatMapM___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Array_allM___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*); @@ -213,11 +233,15 @@ LEAN_EXPORT lean_object* l_Array_instToString(lean_object*); LEAN_EXPORT lean_object* l_Array_reverse___rarg(lean_object*); LEAN_EXPORT lean_object* l_Array_all___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Array_findIdxM_x3f___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_data___rarg(lean_object*); LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at_Array_findSomeRev_x3f___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27_loop___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Array_findIdxM_x3f___spec__1___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_any(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Array_map___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Std_Format_joinSep___at_Array_instRepr___spec__1___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg___lambda__2(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_findSome_x3f___rarg(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_elem___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlM_loop___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -242,12 +266,12 @@ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_forRevM___spec__2( LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_toListImpl___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Array_isEqv___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_appendList(lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_takeWhile___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_ofFn___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_filter___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_allM___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyM_loop___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Array_mapIdx___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at_Array_findSomeRev_x3f___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_indexOf_x3f___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findIdxM_x3f___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); @@ -264,21 +288,25 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe___rarg(lean_object*, lean_object*, l LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Array_findM_x3f___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); static lean_object* l_Array_findSomeM_x3f___rarg___closed__1; LEAN_EXPORT lean_object* l_Array_indexOfAux(lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_insertAt_x21(lean_object*); static lean_object* l_Array_instGetElemUSizeLtNatToNatSize___closed__1; LEAN_EXPORT lean_object* l_Array_back_x3f___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapIdx___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_partition___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findSome_x21___rarg___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapFinIdx___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Array_findIdxM_x3f___spec__1___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_filterM___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at_Array_findRevM_x3f___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_back_x3f___rarg___boxed(lean_object*); lean_object* lean_array_pop(lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___lambda__2(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); static lean_object* l_term_x23_x5b___x2c_x5d___closed__19; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Array_allM___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_findSome_x21___rarg___closed__3; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMap___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMap___spec__1___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Nat_foldTR_loop___at_Array_range___spec__1___at_Array_range___spec__2(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_ofFn_go(lean_object*); @@ -326,17 +354,18 @@ LEAN_EXPORT lean_object* l_Array_filterMapM___rarg___boxed(lean_object*, lean_ob LEAN_EXPORT lean_object* l_Array_zipWith___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_foldr___spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_toListAppend___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdx(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Array_mapIdx___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_modify___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Array_allM___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t); lean_object* l_Lean_Syntax_node2(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapIdxM___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_zipWithAux___at_Array_zip___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_findIdxM_x3f___rarg___closed__1; static lean_object* l_term_x23_x5b___x2c_x5d___closed__1; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapIdxM___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findRevM_x3f___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_toListAppend___spec__2___rarg(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_filter(lean_object*); @@ -360,6 +389,7 @@ LEAN_EXPORT lean_object* l_Array_reverse_loop(lean_object*); static lean_object* l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__11; LEAN_EXPORT lean_object* l_Array_foldl___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Array_allM___spec__2___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_zipWithIndex___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_filterM___spec__1___rarg___lambda__2(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_insertAt(lean_object*); LEAN_EXPORT lean_object* l_Array_eraseIdx___rarg(lean_object*, lean_object*); @@ -372,7 +402,6 @@ LEAN_EXPORT lean_object* l_Array_get_x3f(lean_object*); LEAN_EXPORT lean_object* l_Array_insertAt_loop(lean_object*); LEAN_EXPORT lean_object* l_Array_filterMapM___rarg___lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findSome_x3f(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Array_zipWithIndex___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_instInhabited(lean_object*); LEAN_EXPORT lean_object* l_Array_getEvenElems___rarg___boxed(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -387,18 +416,20 @@ LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___rarg___lambda__1(size_t, lean_ static lean_object* l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__10; LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_pop___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapIdx___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at_Array_instRepr___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Array_erase(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_reduceOption___rarg___boxed(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_getEvenElems___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Array_allM___spec__1___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_term_x23_x5b___x2c_x5d___closed__16; static lean_object* l_term_x23_x5b___x2c_x5d___closed__2; static lean_object* l_term_x23_x5b___x2c_x5d___closed__13; static lean_object* l_Array_instRepr___rarg___closed__3; +LEAN_EXPORT lean_object* l_Array_reduceOption___rarg(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Array_findM_x3f___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_modify___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_term_x23_x5b___x2c_x5d___closed__11; @@ -416,7 +447,9 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_forM___spec__1(lea LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_foldr___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_split___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_take_loop___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forM___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdx___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_filterMapM___at_Array_filterMap___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_any___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -425,11 +458,13 @@ LEAN_EXPORT lean_object* l_Array_filter___rarg___boxed(lean_object*, lean_object LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold(lean_object*, lean_object*, lean_object*); lean_object* l_Array_appendCore___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_filterMap___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapFinIdx___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Array_allM___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_term_x23_x5b___x2c_x5d___closed__8; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Array_findM_x3f___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_reverse_loop___rarg(lean_object*, lean_object*, lean_object*); lean_object* lean_string_length(lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Array_findM_x3f___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -450,6 +485,8 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Array_findIdxM_x3f___spec LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_filterM___spec__1___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_allDiffAux___rarg___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Array_instAppend___closed__1; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapIdxM___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Array_findSome_x3f___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlM_loop___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at_Array_findRevM_x3f___spec__1___rarg___lambda__1(lean_object*, lean_object*, uint8_t); @@ -464,6 +501,7 @@ LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at_Array_findRevM_x3f__ LEAN_EXPORT lean_object* l_Array_instRepr___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Array_map___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_shrink___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMap___spec__1___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_filterM___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Array_takeWhile_go___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_instForIn(lean_object*, lean_object*, lean_object*); @@ -471,6 +509,7 @@ LEAN_EXPORT lean_object* l_Nat_foldTR_loop___at_Array_range___spec__1(lean_objec LEAN_EXPORT lean_object* l_Array_appendList___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Array_insertAt_x21___spec__1___rarg(lean_object*); LEAN_EXPORT lean_object* l_Array_findIdxM_x3f(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___rarg___lambda__1(lean_object*, size_t, lean_object*, lean_object*, size_t, lean_object*); lean_object* l_Lean_Syntax_node1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_getMax_x3f___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_getEvenElems___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); @@ -486,7 +525,6 @@ extern lean_object* l_Id_instMonad; LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f___rarg(lean_object*, lean_object*, lean_object*); lean_object* lean_panic_fn(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_isEqvAux(lean_object*); -LEAN_EXPORT lean_object* l_Array_shrink_loop___rarg(lean_object*, lean_object*); static lean_object* l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__9; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_filterMapM___at_Array_filterMap___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -497,10 +535,10 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Array_findSome_x21___spec LEAN_EXPORT lean_object* l_Array_insertAt_x21___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Array_instRepr___rarg___closed__6; LEAN_EXPORT lean_object* l_Array_toListAppend(lean_object*); -LEAN_EXPORT lean_object* l_Array_shrink_loop(lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_foldr___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_isPrefixOfAux___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_flatMapM___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__17; LEAN_EXPORT lean_object* l_Array_getEvenElems___rarg(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_allDiffAuxAux(lean_object*); @@ -532,6 +570,7 @@ size_t lean_usize_sub(size_t, size_t); LEAN_EXPORT uint8_t l_Array_all___rarg(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_mk(lean_object*); LEAN_EXPORT lean_object* l_Array_takeWhile_go(lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27_loop___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findIdxM_x3f___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_forM___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_modifyOp___rarg(lean_object*, lean_object*, lean_object*); @@ -539,13 +578,18 @@ LEAN_EXPORT lean_object* l_Array_map___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_isPrefixOfAux(lean_object*); size_t lean_usize_add(size_t, size_t); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Array_any___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_flatMap___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at_Array_instRepr___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_instRepr___rarg___closed__7; LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_split___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMap___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_uget(lean_object*, size_t); size_t lean_array_size(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_flatMapM(lean_object*, lean_object*, lean_object*); static lean_object* l_term_x23_x5b___x2c_x5d___closed__6; static lean_object* l_Array_instRepr___rarg___closed__4; LEAN_EXPORT lean_object* l_Array_ofFn_go___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -556,13 +600,18 @@ LEAN_EXPORT lean_object* l_Array_swapAt___rarg___boxed(lean_object*, lean_object LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_toListImpl___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at_Array_findRev_x3f___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Array_all___spec__2(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Array_all___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__15; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_zipWithIndex___spec__1(lean_object*); lean_object* lean_string_append(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_insertAt___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_zipWithIndex___rarg___boxed(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop(lean_object*, lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27_loop___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_shrink___rarg___boxed(lean_object*, lean_object*); static lean_object* l_term_x23_x5b___x2c_x5d___closed__3; LEAN_EXPORT lean_object* l_Array_indexOfAux___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -584,8 +633,9 @@ LEAN_EXPORT lean_object* l_Array_instRepr(lean_object*); static lean_object* l_term_x23_x5b___x2c_x5d___closed__9; LEAN_EXPORT lean_object* l_Array_findIdx_x3f___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_swap___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Array_zipWithIndex___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapIdx___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_zipWith(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapIdxM___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_loop(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrM_fold___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_allM___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -606,14 +656,18 @@ lean_object* lean_array_get(lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__8; lean_object* l___private_Init_Data_Repr_0__Nat_reprFast(lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Array_any___spec__1___rarg(lean_object*, lean_object*, size_t, size_t); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Array_mapIdx___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_allM(lean_object*, lean_object*); static lean_object* l_term_x23_x5b___x2c_x5d___closed__18; LEAN_EXPORT lean_object* l_Array_findSomeM_x3f___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdx___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapIdx___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_popWhile___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_filterM___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_term_x23_x5b___x2c_x5d; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_reduceOption(lean_object*); +LEAN_EXPORT lean_object* l_Array_filterMapM___at_Array_reduceOption___spec__1___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forRevM___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Array_allM___spec__1___rarg___lambda__1(lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Array_anyMUnsafe(lean_object*, lean_object*); @@ -634,6 +688,7 @@ LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___rarg(lean_object*, lean LEAN_EXPORT lean_object* l_Array_modifyMUnsafe___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapM_map___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_isEmpty___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_find_x3f(lean_object*); LEAN_EXPORT lean_object* l_Array_get_x3f___rarg(lean_object*, lean_object*); static lean_object* _init_l_term_x23_x5b___x2c_x5d___closed__1() { @@ -1095,6 +1150,22 @@ return x_34; } } } +LEAN_EXPORT lean_object* l_Array_data___rarg(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_array_to_list(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_data(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_data___rarg), 1, 0); +return x_2; +} +} LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__List_toArrayAux_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { @@ -1127,6 +1198,14 @@ x_3 = lean_alloc_closure((void*)(l___private_Init_Data_Array_Basic_0__List_toArr return x_3; } } +LEAN_EXPORT lean_object* l_Array_instMembership(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_box(0); +return x_2; +} +} LEAN_EXPORT lean_object* l_Array_Array_data___rarg(lean_object* x_1) { _start: { @@ -1791,7 +1870,7 @@ x_9 = l_Array_swapAt_x21___rarg___closed__2; x_10 = lean_string_append(x_8, x_9); x_11 = l_Array_swapAt_x21___rarg___closed__3; x_12 = l_Array_swapAt_x21___rarg___closed__4; -x_13 = lean_unsigned_to_nat(220u); +x_13 = lean_unsigned_to_nat(258u); x_14 = lean_unsigned_to_nat(4u); x_15 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_11, x_12, x_13, x_14, x_10); lean_dec(x_10); @@ -1819,7 +1898,7 @@ x_2 = lean_alloc_closure((void*)(l_Array_swapAt_x21___rarg), 3, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Array_shrink_loop___rarg(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_take_loop___rarg(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; uint8_t x_4; @@ -1843,25 +1922,50 @@ return x_2; } } } -LEAN_EXPORT lean_object* l_Array_shrink_loop(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_take_loop(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Array_shrink_loop___rarg), 2, 0); +x_2 = lean_alloc_closure((void*)(l_Array_take_loop___rarg), 2, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Array_shrink___rarg(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_take___rarg(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; lean_object* x_4; lean_object* x_5; x_3 = lean_array_get_size(x_1); x_4 = lean_nat_sub(x_3, x_2); lean_dec(x_3); -x_5 = l_Array_shrink_loop___rarg(x_4, x_1); +x_5 = l_Array_take_loop___rarg(x_4, x_1); return x_5; } } +LEAN_EXPORT lean_object* l_Array_take(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_take___rarg___boxed), 2, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_take___rarg___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Array_take___rarg(x_1, x_2); +lean_dec(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Array_shrink___rarg(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Array_take___rarg(x_1, x_2); +return x_3; +} +} LEAN_EXPORT lean_object* l_Array_shrink(lean_object* x_1) { _start: { @@ -2276,6 +2380,250 @@ x_4 = lean_alloc_closure((void*)(l_Array_instForIn___rarg), 4, 0); return x_4; } } +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___rarg___lambda__1(lean_object* x_1, size_t x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +if (lean_obj_tag(x_6) == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_4); +lean_dec(x_3); +x_7 = lean_ctor_get(x_6, 0); +lean_inc(x_7); +lean_dec(x_6); +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_2(x_9, lean_box(0), x_7); +return x_10; +} +else +{ +lean_object* x_11; size_t x_12; size_t x_13; lean_object* x_14; +x_11 = lean_ctor_get(x_6, 0); +lean_inc(x_11); +lean_dec(x_6); +x_12 = 1; +x_13 = lean_usize_add(x_2, x_12); +x_14 = l_Array_forIn_x27Unsafe_loop___rarg(x_1, x_3, x_4, x_5, x_13, x_11); +return x_14; +} +} +} +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___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_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_apply_2(x_9, lean_box(0), 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; +x_11 = lean_array_uget(x_2, x_5); +x_12 = lean_ctor_get(x_1, 1); +lean_inc(x_12); +lean_inc(x_3); +x_13 = lean_apply_3(x_3, x_11, lean_box(0), x_6); +x_14 = lean_box_usize(x_5); +x_15 = lean_box_usize(x_4); +x_16 = lean_alloc_closure((void*)(l_Array_forIn_x27Unsafe_loop___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_16, 0, x_1); +lean_closure_set(x_16, 1, x_14); +lean_closure_set(x_16, 2, x_2); +lean_closure_set(x_16, 3, x_3); +lean_closure_set(x_16, 4, x_15); +x_17 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_13, x_16); +return x_17; +} +} +} +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop(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_forIn_x27Unsafe_loop___rarg___boxed), 6, 0); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___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_2); +lean_dec(x_2); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_forIn_x27Unsafe_loop___rarg___lambda__1(x_1, x_7, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___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_forIn_x27Unsafe_loop___rarg(x_1, x_2, x_3, x_7, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe___rarg(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_array_size(x_2); +x_6 = 0; +x_7 = l_Array_forIn_x27Unsafe_loop___rarg(x_1, x_2, x_4, x_5, x_6, x_3); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe(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_forIn_x27Unsafe___rarg), 4, 0); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Array_forIn_x27_loop___rarg___lambda__1(lean_object* x_1, 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_3); +lean_dec(x_2); +x_6 = lean_ctor_get(x_5, 0); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_6); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = l_Array_forIn_x27_loop___rarg(x_1, x_2, x_3, x_4, lean_box(0), x_10); +return x_11; +} +} +} +LEAN_EXPORT lean_object* l_Array_forIn_x27_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) { +_start: +{ +lean_object* x_7; uint8_t x_8; +x_7 = lean_unsigned_to_nat(0u); +x_8 = lean_nat_dec_eq(x_4, x_7); +if (x_8 == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_9 = lean_unsigned_to_nat(1u); +x_10 = lean_nat_sub(x_4, x_9); +x_11 = lean_ctor_get(x_1, 1); +lean_inc(x_11); +x_12 = lean_array_get_size(x_2); +x_13 = lean_nat_sub(x_12, x_9); +lean_dec(x_12); +x_14 = lean_nat_sub(x_13, x_10); +lean_dec(x_13); +x_15 = lean_array_fget(x_2, x_14); +lean_dec(x_14); +lean_inc(x_3); +x_16 = lean_apply_3(x_3, x_15, lean_box(0), x_6); +x_17 = lean_alloc_closure((void*)(l_Array_forIn_x27_loop___rarg___lambda__1___boxed), 5, 4); +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_10); +x_18 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_16, x_17); +return x_18; +} +else +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; +lean_dec(x_3); +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_apply_2(x_20, lean_box(0), x_6); +return x_21; +} +} +} +LEAN_EXPORT lean_object* l_Array_forIn_x27_loop(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_forIn_x27_loop___rarg___boxed), 6, 0); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Array_forIn_x27_loop___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; +x_6 = l_Array_forIn_x27_loop___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_4); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Array_forIn_x27_loop___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; +x_7 = l_Array_forIn_x27_loop___rarg(x_1, x_2, x_3, x_4, x_5, x_6); +lean_dec(x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_instForIn_x27InferInstanceMembership___rarg(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_array_size(x_2); +x_6 = 0; +x_7 = l_Array_forIn_x27Unsafe_loop___rarg(x_1, x_2, x_4, x_5, x_6, x_3); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_instForIn_x27InferInstanceMembership(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_instForIn_x27InferInstanceMembership___rarg), 4, 0); +return x_4; +} +} LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___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: { @@ -2924,18 +3272,18 @@ lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; x_8 = lean_unsigned_to_nat(1u); x_9 = lean_nat_add(x_1, x_8); x_10 = lean_array_push(x_2, x_7); -x_11 = l_Array_mapIdxM_map___rarg(x_3, x_4, x_5, x_6, x_9, lean_box(0), x_10); +x_11 = l_Array_mapFinIdxM_map___rarg(x_3, x_4, x_5, x_6, x_9, lean_box(0), x_10); return x_11; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; uint8_t x_9; @@ -2952,7 +3300,7 @@ x_13 = lean_array_fget(x_2, x_5); lean_inc(x_3); lean_inc(x_5); x_14 = lean_apply_2(x_3, x_5, x_13); -x_15 = lean_alloc_closure((void*)(l_Array_mapIdxM_map___rarg___lambda__1___boxed), 7, 6); +x_15 = lean_alloc_closure((void*)(l_Array_mapFinIdxM_map___rarg___lambda__1___boxed), 7, 6); lean_closure_set(x_15, 0, x_5); lean_closure_set(x_15, 1, x_7); lean_closure_set(x_15, 2, x_1); @@ -2979,33 +3327,118 @@ return x_19; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = lean_alloc_closure((void*)(l_Array_mapFinIdxM_map___rarg___boxed), 7, 0); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; +x_8 = l_Array_mapFinIdxM_map___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_6); +lean_dec(x_1); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; +x_8 = l_Array_mapFinIdxM_map___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_4); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapFinIdxM___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = lean_array_get_size(x_2); +x_5 = lean_mk_empty_array_with_capacity(x_4); +x_6 = lean_unsigned_to_nat(0u); +x_7 = l_Array_mapFinIdxM_map___rarg(x_1, x_2, x_3, x_4, x_6, lean_box(0), x_5); +lean_dec(x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapFinIdxM(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = lean_alloc_closure((void*)(l_Array_mapFinIdxM___rarg), 3, 0); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapIdxM___spec__1___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_9 = lean_unsigned_to_nat(1u); +x_10 = lean_nat_add(x_1, x_9); +x_11 = lean_array_push(x_2, x_8); +x_12 = l_Array_mapFinIdxM_map___at_Array_mapIdxM___spec__1___rarg(x_3, x_4, x_5, x_6, x_7, x_10, lean_box(0), x_11); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapIdxM___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; uint8_t x_10; +x_9 = lean_unsigned_to_nat(0u); +x_10 = lean_nat_dec_eq(x_5, x_9); +if (x_10 == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_11 = lean_unsigned_to_nat(1u); +x_12 = lean_nat_sub(x_5, x_11); +x_13 = lean_ctor_get(x_1, 1); +lean_inc(x_13); +x_14 = lean_array_fget(x_4, x_6); +lean_inc(x_3); +lean_inc(x_6); +x_15 = lean_apply_2(x_3, x_6, x_14); +x_16 = lean_alloc_closure((void*)(l_Array_mapFinIdxM_map___at_Array_mapIdxM___spec__1___rarg___lambda__1___boxed), 8, 7); +lean_closure_set(x_16, 0, x_6); +lean_closure_set(x_16, 1, x_8); +lean_closure_set(x_16, 2, x_1); +lean_closure_set(x_16, 3, x_2); +lean_closure_set(x_16, 4, x_3); +lean_closure_set(x_16, 5, x_4); +lean_closure_set(x_16, 6, x_12); +x_17 = lean_apply_4(x_13, lean_box(0), lean_box(0), x_15, x_16); +return x_17; +} +else +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; +lean_dec(x_6); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_18 = lean_ctor_get(x_1, 0); +lean_inc(x_18); +lean_dec(x_1); +x_19 = lean_ctor_get(x_18, 1); +lean_inc(x_19); +lean_dec(x_18); +x_20 = lean_apply_2(x_19, lean_box(0), x_8); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapIdxM___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = lean_alloc_closure((void*)(l_Array_mapIdxM_map___rarg___boxed), 7, 0); +x_4 = lean_alloc_closure((void*)(l_Array_mapFinIdxM_map___at_Array_mapIdxM___spec__1___rarg___boxed), 8, 0); return x_4; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; -x_8 = l_Array_mapIdxM_map___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -lean_dec(x_6); -lean_dec(x_1); -return x_8; -} -} -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; -x_8 = l_Array_mapIdxM_map___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -lean_dec(x_4); -return x_8; -} -} LEAN_EXPORT lean_object* l_Array_mapIdxM___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { @@ -3013,7 +3446,8 @@ lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_4 = lean_array_get_size(x_2); x_5 = lean_mk_empty_array_with_capacity(x_4); x_6 = lean_unsigned_to_nat(0u); -x_7 = l_Array_mapIdxM_map___rarg(x_1, x_2, x_3, x_4, x_6, lean_box(0), x_5); +lean_inc(x_2); +x_7 = l_Array_mapFinIdxM_map___at_Array_mapIdxM___spec__1___rarg(x_1, x_2, x_3, x_2, x_4, x_6, lean_box(0), x_5); lean_dec(x_4); return x_7; } @@ -3026,6 +3460,25 @@ x_4 = lean_alloc_closure((void*)(l_Array_mapIdxM___rarg), 3, 0); return x_4; } } +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapIdxM___spec__1___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +x_9 = l_Array_mapFinIdxM_map___at_Array_mapIdxM___spec__1___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_7); +lean_dec(x_1); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapIdxM___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +x_9 = l_Array_mapFinIdxM_map___at_Array_mapIdxM___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_5); +return x_9; +} +} LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Array_findSomeM_x3f___spec__1___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { @@ -5532,7 +5985,87 @@ x_7 = l_Array_mapMUnsafe_map___at_Array_map___spec__1___rarg(x_1, x_5, x_6, x_4) return x_7; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Array_mapIdx___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapFinIdx___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; uint8_t x_9; +x_8 = lean_unsigned_to_nat(0u); +x_9 = lean_nat_dec_eq(x_4, x_8); +if (x_9 == 0) +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_10 = lean_unsigned_to_nat(1u); +x_11 = lean_nat_sub(x_4, x_10); +lean_dec(x_4); +x_12 = lean_array_fget(x_3, x_5); +lean_inc(x_2); +lean_inc(x_5); +x_13 = lean_apply_2(x_2, x_5, x_12); +x_14 = lean_nat_add(x_5, x_10); +lean_dec(x_5); +x_15 = lean_array_push(x_7, x_13); +x_4 = x_11; +x_5 = x_14; +x_6 = lean_box(0); +x_7 = x_15; +goto _start; +} +else +{ +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +return x_7; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapFinIdx___spec__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Array_mapFinIdxM_map___at_Array_mapFinIdx___spec__1___rarg___boxed), 7, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Array_mapFinIdx___rarg(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_3 = lean_array_get_size(x_1); +x_4 = lean_mk_empty_array_with_capacity(x_3); +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Array_mapFinIdxM_map___at_Array_mapFinIdx___spec__1___rarg(x_1, x_2, x_1, x_3, x_5, lean_box(0), x_4); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Array_mapFinIdx(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Array_mapFinIdx___rarg___boxed), 2, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapFinIdx___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; +x_8 = l_Array_mapFinIdxM_map___at_Array_mapFinIdx___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_3); +lean_dec(x_1); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapFinIdx___rarg___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Array_mapFinIdx___rarg(x_1, x_2); +lean_dec(x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapIdx___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; uint8_t x_9; @@ -5566,11 +6099,11 @@ return x_7; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Array_mapIdx___spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapIdx___spec__1(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Array_mapIdxM_map___at_Array_mapIdx___spec__1___rarg___boxed), 7, 0); +x_3 = lean_alloc_closure((void*)(l_Array_mapFinIdxM_map___at_Array_mapIdx___spec__1___rarg___boxed), 7, 0); return x_3; } } @@ -5581,7 +6114,7 @@ lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_3 = lean_array_get_size(x_1); x_4 = lean_mk_empty_array_with_capacity(x_3); x_5 = lean_unsigned_to_nat(0u); -x_6 = l_Array_mapIdxM_map___at_Array_mapIdx___spec__1___rarg(x_1, x_2, x_1, x_3, x_5, lean_box(0), x_4); +x_6 = l_Array_mapFinIdxM_map___at_Array_mapIdx___spec__1___rarg(x_1, x_2, x_1, x_3, x_5, lean_box(0), x_4); return x_6; } } @@ -5593,11 +6126,11 @@ x_3 = lean_alloc_closure((void*)(l_Array_mapIdx___rarg___boxed), 2, 0); return x_3; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Array_mapIdx___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapIdx___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; -x_8 = l_Array_mapIdxM_map___at_Array_mapIdx___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Array_mapFinIdxM_map___at_Array_mapIdx___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_3); lean_dec(x_1); return x_8; @@ -5612,7 +6145,7 @@ lean_dec(x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Array_zipWithIndex___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_zipWithIndex___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; uint8_t x_8; @@ -5646,11 +6179,11 @@ return x_6; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Array_zipWithIndex___spec__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_zipWithIndex___spec__1(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Array_mapIdxM_map___at_Array_zipWithIndex___spec__1___rarg___boxed), 6, 0); +x_2 = lean_alloc_closure((void*)(l_Array_mapFinIdxM_map___at_Array_zipWithIndex___spec__1___rarg___boxed), 6, 0); return x_2; } } @@ -5661,7 +6194,7 @@ lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_2 = lean_array_get_size(x_1); x_3 = lean_mk_empty_array_with_capacity(x_2); x_4 = lean_unsigned_to_nat(0u); -x_5 = l_Array_mapIdxM_map___at_Array_zipWithIndex___spec__1___rarg(x_1, x_1, x_2, x_4, lean_box(0), x_3); +x_5 = l_Array_mapFinIdxM_map___at_Array_zipWithIndex___spec__1___rarg(x_1, x_1, x_2, x_4, lean_box(0), x_3); return x_5; } } @@ -5673,11 +6206,11 @@ x_2 = lean_alloc_closure((void*)(l_Array_zipWithIndex___rarg___boxed), 1, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Array_zipWithIndex___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_zipWithIndex___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; -x_7 = l_Array_mapIdxM_map___at_Array_zipWithIndex___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Array_mapFinIdxM_map___at_Array_zipWithIndex___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_2); lean_dec(x_1); return x_7; @@ -6074,7 +6607,7 @@ static lean_object* _init_l_Array_findSome_x21___rarg___closed__3() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Array_swapAt_x21___rarg___closed__3; x_2 = l_Array_findSome_x21___rarg___closed__1; -x_3 = lean_unsigned_to_nat(538u); +x_3 = lean_unsigned_to_nat(620u); x_4 = lean_unsigned_to_nat(14u); x_5 = l_Array_findSome_x21___rarg___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -7512,54 +8045,215 @@ x_2 = lean_alloc_closure((void*)(l_List_foldl___at_Array_appendList___spec__1___ return x_2; } } -LEAN_EXPORT lean_object* l_Array_appendList___rarg(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = l_List_foldl___at_Array_appendList___spec__1___rarg(x_1, x_2); -return x_3; +LEAN_EXPORT lean_object* l_Array_appendList___rarg(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_List_foldl___at_Array_appendList___spec__1___rarg(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Array_appendList(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_appendList___rarg), 2, 0); +return x_2; +} +} +static lean_object* _init_l_Array_instHAppendList___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Array_appendList___rarg), 2, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Array_instHAppendList(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = l_Array_instHAppendList___closed__1; +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +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_Array_append___rarg(x_2, x_3); +x_7 = lean_apply_2(x_5, lean_box(0), x_6); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg___lambda__2(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg(x_2, x_3, x_4, x_8, x_5, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6) { +_start: +{ +uint8_t x_7; +x_7 = lean_usize_dec_eq(x_4, x_5); +if (x_7 == 0) +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_8 = lean_ctor_get(x_1, 1); +lean_inc(x_8); +x_9 = lean_array_uget(x_3, x_4); +lean_inc(x_2); +x_10 = lean_apply_1(x_2, x_9); +lean_inc(x_1); +x_11 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg___lambda__1___boxed), 3, 2); +lean_closure_set(x_11, 0, x_1); +lean_closure_set(x_11, 1, x_6); +lean_inc(x_8); +x_12 = lean_apply_4(x_8, lean_box(0), lean_box(0), x_10, x_11); +x_13 = lean_box_usize(x_4); +x_14 = lean_box_usize(x_5); +x_15 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg___lambda__2___boxed), 6, 5); +lean_closure_set(x_15, 0, x_13); +lean_closure_set(x_15, 1, x_1); +lean_closure_set(x_15, 2, x_2); +lean_closure_set(x_15, 3, x_3); +lean_closure_set(x_15, 4, x_14); +x_16 = lean_apply_4(x_8, lean_box(0), lean_box(0), x_12, x_15); +return x_16; +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +lean_dec(x_3); +lean_dec(x_2); +x_17 = lean_ctor_get(x_1, 0); +lean_inc(x_17); +lean_dec(x_1); +x_18 = lean_ctor_get(x_17, 1); +lean_inc(x_18); +lean_dec(x_17); +x_19 = lean_apply_2(x_18, lean_box(0), x_6); +return x_19; +} +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg___boxed), 6, 0); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Array_flatMapM___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; uint8_t x_6; +x_4 = lean_array_get_size(x_3); +x_5 = lean_unsigned_to_nat(0u); +x_6 = lean_nat_dec_lt(x_5, x_4); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__18; +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +uint8_t x_11; +x_11 = lean_nat_dec_le(x_4, x_4); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_12 = lean_ctor_get(x_1, 0); +lean_inc(x_12); +lean_dec(x_1); +x_13 = lean_ctor_get(x_12, 1); +lean_inc(x_13); +lean_dec(x_12); +x_14 = l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__18; +x_15 = lean_apply_2(x_13, lean_box(0), x_14); +return x_15; +} +else +{ +size_t x_16; size_t x_17; lean_object* x_18; lean_object* x_19; +x_16 = 0; +x_17 = lean_usize_of_nat(x_4); +lean_dec(x_4); +x_18 = l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__18; +x_19 = l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg(x_1, x_2, x_3, x_16, x_17, x_18); +return x_19; +} +} } } -LEAN_EXPORT lean_object* l_Array_appendList(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_flatMapM(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Array_appendList___rarg), 2, 0); -return x_2; +lean_object* x_4; +x_4 = lean_alloc_closure((void*)(l_Array_flatMapM___rarg), 3, 0); +return x_4; } } -static lean_object* _init_l_Array_instHAppendList___closed__1() { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Array_appendList___rarg), 2, 0); -return x_1; +lean_object* x_4; +x_4 = l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg___lambda__1(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; } } -LEAN_EXPORT lean_object* l_Array_instHAppendList(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { -lean_object* x_2; -x_2 = l_Array_instHAppendList___closed__1; -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_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg___lambda__2(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg___boxed(lean_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_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); +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_4); lean_dec(x_4); -x_6 = l_Array_append___rarg(x_2, x_3); -x_7 = lean_apply_2(x_5, lean_box(0), x_6); -return x_7; +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg(x_1, x_2, x_3, x_7, x_8, x_6); +return x_9; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___lambda__2(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { _start: { size_t x_7; size_t x_8; lean_object* x_9; @@ -7583,14 +8277,14 @@ x_9 = lean_array_uget(x_3, x_4); lean_inc(x_2); x_10 = lean_apply_1(x_2, x_9); lean_inc(x_1); -x_11 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___lambda__1___boxed), 3, 2); +x_11 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg___lambda__1___boxed), 3, 2); lean_closure_set(x_11, 0, x_1); lean_closure_set(x_11, 1, x_6); lean_inc(x_8); x_12 = lean_apply_4(x_8, lean_box(0), lean_box(0), x_10, x_11); x_13 = lean_box_usize(x_4); x_14 = lean_box_usize(x_5); -x_15 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___lambda__2___boxed), 6, 5); +x_15 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___lambda__1___boxed), 6, 5); lean_closure_set(x_15, 0, x_13); lean_closure_set(x_15, 1, x_1); lean_closure_set(x_15, 2, x_2); @@ -7687,16 +8381,7 @@ x_4 = lean_alloc_closure((void*)(l_Array_concatMapM___rarg), 3, 0); return x_4; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___lambda__1(x_1, x_2, x_3); -lean_dec(x_3); -return x_4; -} -} -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { size_t x_7; size_t x_8; lean_object* x_9; @@ -7704,7 +8389,7 @@ x_7 = lean_unbox_usize(x_1); lean_dec(x_1); x_8 = lean_unbox_usize(x_5); lean_dec(x_5); -x_9 = l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___lambda__2(x_7, x_2, x_3, x_4, x_8, x_6); +x_9 = l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); return x_9; } } @@ -7720,6 +8405,110 @@ x_9 = l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg(x_1, x_2, return x_9; } } +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMap___spec__1___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_eq(x_3, x_4); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; size_t x_10; size_t x_11; +x_7 = lean_array_uget(x_2, x_3); +lean_inc(x_1); +x_8 = lean_apply_1(x_1, x_7); +x_9 = l_Array_append___rarg(x_5, x_8); +lean_dec(x_8); +x_10 = 1; +x_11 = lean_usize_add(x_3, x_10); +x_3 = x_11; +x_5 = x_9; +goto _start; +} +else +{ +lean_dec(x_1); +return x_5; +} +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMap___spec__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Array_flatMap___spec__1___rarg___boxed), 5, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Array_flatMap___rarg(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; uint8_t x_5; +x_3 = lean_array_get_size(x_2); +x_4 = lean_unsigned_to_nat(0u); +x_5 = lean_nat_dec_lt(x_4, x_3); +if (x_5 == 0) +{ +lean_object* x_6; +lean_dec(x_3); +lean_dec(x_1); +x_6 = l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__18; +return x_6; +} +else +{ +uint8_t x_7; +x_7 = lean_nat_dec_le(x_3, x_3); +if (x_7 == 0) +{ +lean_object* x_8; +lean_dec(x_3); +lean_dec(x_1); +x_8 = l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__18; +return x_8; +} +else +{ +size_t x_9; size_t x_10; lean_object* x_11; lean_object* x_12; +x_9 = 0; +x_10 = lean_usize_of_nat(x_3); +lean_dec(x_3); +x_11 = l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__18; +x_12 = l_Array_foldlMUnsafe_fold___at_Array_flatMap___spec__1___rarg(x_1, x_2, x_9, x_10, x_11); +return x_12; +} +} +} +} +LEAN_EXPORT lean_object* l_Array_flatMap(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Array_flatMap___rarg___boxed), 2, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMap___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_foldlMUnsafe_fold___at_Array_flatMap___spec__1___rarg(x_1, x_2, x_6, x_7, x_5); +lean_dec(x_2); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_flatMap___rarg___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Array_flatMap___rarg(x_1, x_2); +lean_dec(x_2); +return x_3; +} +} LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMap___spec__1___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { _start: { @@ -9174,7 +9963,7 @@ static lean_object* _init_l_Array_insertAt_x21___rarg___closed__3() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Array_swapAt_x21___rarg___closed__3; x_2 = l_Array_insertAt_x21___rarg___closed__1; -x_3 = lean_unsigned_to_nat(764u); +x_3 = lean_unsigned_to_nat(850u); x_4 = lean_unsigned_to_nat(7u); x_5 = l_Array_insertAt_x21___rarg___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -9814,6 +10603,143 @@ lean_dec(x_1); return x_3; } } +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_reduceOption___spec__2___rarg(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; +x_5 = lean_usize_dec_eq(x_2, x_3); +if (x_5 == 0) +{ +lean_object* x_6; size_t x_7; size_t x_8; +x_6 = lean_array_uget(x_1, x_2); +x_7 = 1; +x_8 = lean_usize_add(x_2, x_7); +if (lean_obj_tag(x_6) == 0) +{ +x_2 = x_8; +goto _start; +} +else +{ +lean_object* x_10; lean_object* x_11; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_array_push(x_4, x_10); +x_2 = x_8; +x_4 = x_11; +goto _start; +} +} +else +{ +return x_4; +} +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_reduceOption___spec__2(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Array_reduceOption___spec__2___rarg___boxed), 4, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_filterMapM___at_Array_reduceOption___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +uint8_t x_4; +x_4 = lean_nat_dec_lt(x_2, x_3); +if (x_4 == 0) +{ +lean_object* x_5; +x_5 = l_Array_filter___rarg___closed__1; +return x_5; +} +else +{ +lean_object* x_6; uint8_t x_7; +x_6 = lean_array_get_size(x_1); +x_7 = lean_nat_dec_le(x_3, x_6); +lean_dec(x_6); +if (x_7 == 0) +{ +lean_object* x_8; +x_8 = l_Array_filter___rarg___closed__1; +return x_8; +} +else +{ +size_t x_9; size_t x_10; lean_object* x_11; lean_object* x_12; +x_9 = lean_usize_of_nat(x_2); +x_10 = lean_usize_of_nat(x_3); +x_11 = l_Array_filter___rarg___closed__1; +x_12 = l_Array_foldlMUnsafe_fold___at_Array_reduceOption___spec__2___rarg(x_1, x_9, x_10, x_11); +return x_12; +} +} +} +} +LEAN_EXPORT lean_object* l_Array_filterMapM___at_Array_reduceOption___spec__1(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_filterMapM___at_Array_reduceOption___spec__1___rarg___boxed), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_reduceOption___rarg(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_2 = lean_array_get_size(x_1); +x_3 = lean_unsigned_to_nat(0u); +x_4 = l_Array_filterMapM___at_Array_reduceOption___spec__1___rarg(x_1, x_3, x_2); +lean_dec(x_2); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Array_reduceOption(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_reduceOption___rarg___boxed), 1, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_reduceOption___spec__2___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_foldlMUnsafe_fold___at_Array_reduceOption___spec__2___rarg(x_1, x_5, x_6, x_4); +lean_dec(x_1); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_filterMapM___at_Array_reduceOption___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Array_filterMapM___at_Array_reduceOption___spec__1___rarg(x_1, x_2, x_3); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Array_reduceOption___rarg___boxed(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = l_Array_reduceOption___rarg(x_1); +lean_dec(x_1); +return x_2; +} +} LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_eraseReps___spec__1___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { _start: { diff --git a/stage0/stdlib/Init/Data/Array/DecidableEq.c b/stage0/stdlib/Init/Data/Array/DecidableEq.c index 2ddc56fdb3bc..d0515e31b318 100644 --- a/stage0/stdlib/Init/Data/Array/DecidableEq.c +++ b/stage0/stdlib/Init/Data/Array/DecidableEq.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Init.Data.Array.DecidableEq -// Imports: Init.Data.Array.Basic Init.Data.BEq Init.ByCases +// Imports: Init.Data.Array.Basic Init.Data.BEq Init.Data.Nat.Lemmas Init.Data.List.Nat.BEq Init.ByCases #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -187,6 +187,8 @@ return x_5; } lean_object* initialize_Init_Data_Array_Basic(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_BEq(uint8_t builtin, lean_object*); +lean_object* initialize_Init_Data_Nat_Lemmas(uint8_t builtin, lean_object*); +lean_object* initialize_Init_Data_List_Nat_BEq(uint8_t builtin, lean_object*); lean_object* initialize_Init_ByCases(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Init_Data_Array_DecidableEq(uint8_t builtin, lean_object* w) { @@ -199,6 +201,12 @@ lean_dec_ref(res); res = initialize_Init_Data_BEq(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +res = initialize_Init_Data_Nat_Lemmas(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Init_Data_List_Nat_BEq(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); res = initialize_Init_ByCases(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Init/Data/Array/GetLit.c b/stage0/stdlib/Init/Data/Array/GetLit.c index 03fb16fcacd4..6da8fc3d154d 100644 --- a/stage0/stdlib/Init/Data/Array/GetLit.c +++ b/stage0/stdlib/Init/Data/Array/GetLit.c @@ -145,56 +145,6 @@ lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l___private_Init_Data_Array_GetLit_0__Array_toListLitAux_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; uint8_t x_7; -x_6 = lean_unsigned_to_nat(0u); -x_7 = lean_nat_dec_eq(x_1, x_6); -if (x_7 == 0) -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; -lean_dec(x_4); -x_8 = lean_unsigned_to_nat(1u); -x_9 = lean_nat_sub(x_1, x_8); -x_10 = lean_apply_3(x_5, x_9, lean_box(0), x_3); -return x_10; -} -else -{ -lean_object* x_11; -lean_dec(x_5); -x_11 = lean_apply_2(x_4, lean_box(0), x_3); -return x_11; -} -} -} -LEAN_EXPORT lean_object* l___private_Init_Data_Array_GetLit_0__Array_toListLitAux_match__1_splitter(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = lean_alloc_closure((void*)(l___private_Init_Data_Array_GetLit_0__Array_toListLitAux_match__1_splitter___rarg___boxed), 5, 0); -return x_4; -} -} -LEAN_EXPORT lean_object* l___private_Init_Data_Array_GetLit_0__Array_toListLitAux_match__1_splitter___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; -x_6 = l___private_Init_Data_Array_GetLit_0__Array_toListLitAux_match__1_splitter___rarg(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_1); -return x_6; -} -} -LEAN_EXPORT lean_object* l___private_Init_Data_Array_GetLit_0__Array_toListLitAux_match__1_splitter___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l___private_Init_Data_Array_GetLit_0__Array_toListLitAux_match__1_splitter(x_1, x_2, x_3); -lean_dec(x_2); -return x_4; -} -} LEAN_EXPORT lean_object* l___private_Init_Data_Array_GetLit_0__List_take_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { @@ -254,6 +204,56 @@ lean_dec(x_1); return x_6; } } +LEAN_EXPORT lean_object* l___private_Init_Data_Array_GetLit_0__Array_toListLitAux_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; uint8_t x_7; +x_6 = lean_unsigned_to_nat(0u); +x_7 = lean_nat_dec_eq(x_1, x_6); +if (x_7 == 0) +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_4); +x_8 = lean_unsigned_to_nat(1u); +x_9 = lean_nat_sub(x_1, x_8); +x_10 = lean_apply_3(x_5, x_9, lean_box(0), x_3); +return x_10; +} +else +{ +lean_object* x_11; +lean_dec(x_5); +x_11 = lean_apply_2(x_4, lean_box(0), x_3); +return x_11; +} +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Array_GetLit_0__Array_toListLitAux_match__1_splitter(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = lean_alloc_closure((void*)(l___private_Init_Data_Array_GetLit_0__Array_toListLitAux_match__1_splitter___rarg___boxed), 5, 0); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Array_GetLit_0__Array_toListLitAux_match__1_splitter___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; +x_6 = l___private_Init_Data_Array_GetLit_0__Array_toListLitAux_match__1_splitter___rarg(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_1); +return x_6; +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Array_GetLit_0__Array_toListLitAux_match__1_splitter___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Init_Data_Array_GetLit_0__Array_toListLitAux_match__1_splitter(x_1, x_2, x_3); +lean_dec(x_2); +return x_4; +} +} lean_object* initialize_Init_Data_Array_Basic(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Init_Data_Array_GetLit(uint8_t builtin, lean_object* w) { diff --git a/stage0/stdlib/Init/Data/Array/Lemmas.c b/stage0/stdlib/Init/Data/Array/Lemmas.c index 6c9aa1689e37..895d318cae9c 100644 --- a/stage0/stdlib/Init/Data/Array/Lemmas.c +++ b/stage0/stdlib/Init/Data/Array/Lemmas.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Init.Data.Array.Lemmas -// Imports: Init.Data.Nat.Lemmas Init.Data.List.Impl Init.Data.List.Monadic Init.Data.List.Range Init.Data.Array.Mem Init.TacticsExtra +// Imports: Init.Data.Nat.Lemmas Init.Data.List.Impl Init.Data.List.Monadic Init.Data.List.Range Init.Data.List.Nat.TakeDrop Init.Data.List.Nat.Modify Init.Data.Array.Mem Init.TacticsExtra #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -13,20 +13,24 @@ #ifdef __cplusplus extern "C" { #endif +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_take_loop_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_findSomeRevM_x3f_find_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_findSomeRevM_x3f_find_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_toListRev___rarg___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_foldlM_loop_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_mapIdxM_map_match__1_splitter(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_toListRev___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Array_instDecidableMemOfDecidableEq___spec__2(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_isEqvAux_match__1_splitter___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__GetElem_x3f_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__List_forIn_loop_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__List_anyM_match__1_splitter___rarg(uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Array_instDecidableMemOfDecidableEq___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_take_loop_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_isEqvAux_match__1_splitter(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_appendCore_loop_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__List_forIn_x27__cons_match__1_splitter(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_foldlM_loop_match__1_splitter(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__List_filterMap_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_instDecidableMemOfDecidableEq(lean_object*); @@ -40,18 +44,22 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_toListRev___spec__ LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Nat_fold_match__1_splitter(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_isEqvAux_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Nat_fold_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__List_forIn_x27__cons_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_forInUnsafe_loop_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_isEqvAux_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_take_loop_match__1_splitter(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_findSomeRevM_x3f_find_match__1_splitter(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_toListRev___spec__1(lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_forInUnsafe_loop_match__1_splitter(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__List_anyM_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_foldlM_loop_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_mapIdxM_map_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_mapIdxM_map_match__1_splitter___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__List_forIn_loop_match__1_splitter(lean_object*, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Array_instDecidableMemOfDecidableEq___spec__2___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t); lean_object* lean_nat_sub(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__List_anyM_match__1_splitter(lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__GetElem_x3f_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_appendCore_loop_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); LEAN_EXPORT lean_object* l_Array_instDecidableMemOfDecidableEq___rarg___boxed(lean_object*, lean_object*, lean_object*); @@ -59,10 +67,196 @@ lean_object* lean_array_uget(lean_object*, size_t); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Nat_fold_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_instDecidableMemOfDecidableEq___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_toListRev(lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_mapIdxM_map_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_contains___at_Array_instDecidableMemOfDecidableEq___spec__1___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__GetElem_x3f_match__1_splitter(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__GetElem_x3f_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_dec(x_2); +lean_inc(x_3); +return x_3; +} +else +{ +lean_object* x_4; lean_object* x_5; +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_apply_1(x_2, x_4); +return x_5; +} +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__GetElem_x3f_match__1_splitter(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l___private_Init_Data_Array_Lemmas_0__GetElem_x3f_match__1_splitter___rarg___boxed), 3, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__GetElem_x3f_match__1_splitter___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Init_Data_Array_Lemmas_0__GetElem_x3f_match__1_splitter___rarg(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_isEqvAux_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; uint8_t x_6; +x_5 = lean_unsigned_to_nat(0u); +x_6 = lean_nat_dec_eq(x_1, x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_dec(x_3); +x_7 = lean_unsigned_to_nat(1u); +x_8 = lean_nat_sub(x_1, x_7); +x_9 = lean_apply_2(x_4, x_8, lean_box(0)); +return x_9; +} +else +{ +lean_object* x_10; +lean_dec(x_4); +x_10 = lean_apply_1(x_3, lean_box(0)); +return x_10; +} +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_isEqvAux_match__1_splitter(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = lean_alloc_closure((void*)(l___private_Init_Data_Array_Lemmas_0__Array_isEqvAux_match__1_splitter___rarg___boxed), 4, 0); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_isEqvAux_match__1_splitter___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l___private_Init_Data_Array_Lemmas_0__Array_isEqvAux_match__1_splitter___rarg(x_1, x_2, x_3, x_4); +lean_dec(x_1); +return x_5; +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_isEqvAux_match__1_splitter___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Init_Data_Array_Lemmas_0__Array_isEqvAux_match__1_splitter(x_1, x_2, x_3); +lean_dec(x_2); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_forInUnsafe_loop_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_4; lean_object* x_5; +lean_dec(x_3); +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_apply_1(x_2, x_4); +return x_5; +} +else +{ +lean_object* x_6; lean_object* x_7; +lean_dec(x_2); +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +lean_dec(x_1); +x_7 = lean_apply_1(x_3, x_6); +return x_7; +} +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_forInUnsafe_loop_match__1_splitter(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l___private_Init_Data_Array_Lemmas_0__Array_forInUnsafe_loop_match__1_splitter___rarg), 3, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__List_forIn_loop_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_4; lean_object* x_5; +lean_dec(x_3); +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_apply_1(x_2, x_4); +return x_5; +} +else +{ +lean_object* x_6; lean_object* x_7; +lean_dec(x_2); +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +lean_dec(x_1); +x_7 = lean_apply_1(x_3, x_6); +return x_7; +} +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__List_forIn_loop_match__1_splitter(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l___private_Init_Data_Array_Lemmas_0__List_forIn_loop_match__1_splitter___rarg), 3, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__List_forIn_x27__cons_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_4; lean_object* x_5; +lean_dec(x_3); +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_apply_1(x_2, x_4); +return x_5; +} +else +{ +lean_object* x_6; lean_object* x_7; +lean_dec(x_2); +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +lean_dec(x_1); +x_7 = lean_apply_1(x_3, x_6); +return x_7; +} +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__List_forIn_x27__cons_match__1_splitter(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l___private_Init_Data_Array_Lemmas_0__List_forIn_x27__cons_match__1_splitter___rarg), 3, 0); +return x_3; +} +} LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_toListRev___spec__1___rarg(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { @@ -200,47 +394,7 @@ lean_dec(x_1); return x_5; } } -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_foldlM_loop_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; uint8_t x_5; -x_4 = lean_unsigned_to_nat(0u); -x_5 = lean_nat_dec_eq(x_1, x_4); -if (x_5 == 0) -{ -lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_6 = lean_unsigned_to_nat(1u); -x_7 = lean_nat_sub(x_1, x_6); -x_8 = lean_apply_1(x_3, x_7); -return x_8; -} -else -{ -lean_dec(x_3); -lean_inc(x_2); -return x_2; -} -} -} -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_foldlM_loop_match__1_splitter(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l___private_Init_Data_Array_Lemmas_0__Array_foldlM_loop_match__1_splitter___rarg___boxed), 3, 0); -return x_2; -} -} -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_foldlM_loop_match__1_splitter___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l___private_Init_Data_Array_Lemmas_0__Array_foldlM_loop_match__1_splitter___rarg(x_1, x_2, x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_4; -} -} -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_isEqvAux_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_take_loop_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; uint8_t x_6; @@ -252,93 +406,73 @@ lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_dec(x_3); x_7 = lean_unsigned_to_nat(1u); x_8 = lean_nat_sub(x_1, x_7); -x_9 = lean_apply_2(x_4, x_8, lean_box(0)); +x_9 = lean_apply_2(x_4, x_8, x_2); return x_9; } else { lean_object* x_10; lean_dec(x_4); -x_10 = lean_apply_1(x_3, lean_box(0)); +x_10 = lean_apply_1(x_3, x_2); return x_10; } } } -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_isEqvAux_match__1_splitter(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_take_loop_match__1_splitter(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_4; -x_4 = lean_alloc_closure((void*)(l___private_Init_Data_Array_Lemmas_0__Array_isEqvAux_match__1_splitter___rarg___boxed), 4, 0); -return x_4; +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l___private_Init_Data_Array_Lemmas_0__Array_take_loop_match__1_splitter___rarg___boxed), 4, 0); +return x_3; } } -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_isEqvAux_match__1_splitter___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_take_loop_match__1_splitter___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l___private_Init_Data_Array_Lemmas_0__Array_isEqvAux_match__1_splitter___rarg(x_1, x_2, x_3, x_4); +x_5 = l___private_Init_Data_Array_Lemmas_0__Array_take_loop_match__1_splitter___rarg(x_1, x_2, x_3, x_4); lean_dec(x_1); return x_5; } } -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_isEqvAux_match__1_splitter___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l___private_Init_Data_Array_Lemmas_0__Array_isEqvAux_match__1_splitter(x_1, x_2, x_3); -lean_dec(x_2); -return x_4; -} -} -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_mapIdxM_map_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_foldlM_loop_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_5; uint8_t x_6; -x_5 = lean_unsigned_to_nat(0u); -x_6 = lean_nat_dec_eq(x_1, x_5); -if (x_6 == 0) +lean_object* x_4; uint8_t x_5; +x_4 = lean_unsigned_to_nat(0u); +x_5 = lean_nat_dec_eq(x_1, x_4); +if (x_5 == 0) { -lean_object* x_7; lean_object* x_8; lean_object* x_9; -lean_dec(x_3); -x_7 = lean_unsigned_to_nat(1u); -x_8 = lean_nat_sub(x_1, x_7); -x_9 = lean_apply_2(x_4, x_8, lean_box(0)); -return x_9; +lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_6 = lean_unsigned_to_nat(1u); +x_7 = lean_nat_sub(x_1, x_6); +x_8 = lean_apply_1(x_3, x_7); +return x_8; } else { -lean_object* x_10; -lean_dec(x_4); -x_10 = lean_apply_1(x_3, lean_box(0)); -return x_10; -} -} +lean_dec(x_3); +lean_inc(x_2); +return x_2; } -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_mapIdxM_map_match__1_splitter(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -lean_object* x_5; -x_5 = lean_alloc_closure((void*)(l___private_Init_Data_Array_Lemmas_0__Array_mapIdxM_map_match__1_splitter___rarg___boxed), 4, 0); -return x_5; } } -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_mapIdxM_map_match__1_splitter___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_foldlM_loop_match__1_splitter(lean_object* x_1) { _start: { -lean_object* x_5; -x_5 = l___private_Init_Data_Array_Lemmas_0__Array_mapIdxM_map_match__1_splitter___rarg(x_1, x_2, x_3, x_4); -lean_dec(x_1); -return x_5; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l___private_Init_Data_Array_Lemmas_0__Array_foldlM_loop_match__1_splitter___rarg___boxed), 3, 0); +return x_2; } } -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_mapIdxM_map_match__1_splitter___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_foldlM_loop_match__1_splitter___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_5; -x_5 = l___private_Init_Data_Array_Lemmas_0__Array_mapIdxM_map_match__1_splitter(x_1, x_2, x_3, x_4); -lean_dec(x_3); +lean_object* x_4; +x_4 = l___private_Init_Data_Array_Lemmas_0__Array_foldlM_loop_match__1_splitter___rarg(x_1, x_2, x_3); lean_dec(x_2); -return x_5; +lean_dec(x_1); +return x_4; } } LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_findSomeRevM_x3f_find_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { @@ -628,6 +762,8 @@ lean_object* initialize_Init_Data_Nat_Lemmas(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_List_Impl(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_List_Monadic(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_List_Range(uint8_t builtin, lean_object*); +lean_object* initialize_Init_Data_List_Nat_TakeDrop(uint8_t builtin, lean_object*); +lean_object* initialize_Init_Data_List_Nat_Modify(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_Array_Mem(uint8_t builtin, lean_object*); lean_object* initialize_Init_TacticsExtra(uint8_t builtin, lean_object*); static bool _G_initialized = false; @@ -647,6 +783,12 @@ lean_dec_ref(res); res = initialize_Init_Data_List_Range(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +res = initialize_Init_Data_List_Nat_TakeDrop(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Init_Data_List_Nat_Modify(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); res = initialize_Init_Data_Array_Mem(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Init/Data/Array/MapIdx.c b/stage0/stdlib/Init/Data/Array/MapIdx.c new file mode 100644 index 000000000000..9f2d423744f9 --- /dev/null +++ b/stage0/stdlib/Init/Data/Array/MapIdx.c @@ -0,0 +1,90 @@ +// Lean compiler output +// Module: Init.Data.Array.MapIdx +// Imports: Init.Data.Array.Lemmas Init.Data.List.MapIdx +#include +#if defined(__clang__) +#pragma clang diagnostic ignored "-Wunused-parameter" +#pragma clang diagnostic ignored "-Wunused-label" +#elif defined(__GNUC__) && !defined(__CLANG__) +#pragma GCC diagnostic ignored "-Wunused-parameter" +#pragma GCC diagnostic ignored "-Wunused-label" +#pragma GCC diagnostic ignored "-Wunused-but-set-variable" +#endif +#ifdef __cplusplus +extern "C" { +#endif +LEAN_EXPORT lean_object* l___private_Init_Data_Array_MapIdx_0__Array_mapFinIdxM_map_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Array_MapIdx_0__Array_mapFinIdxM_map_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Array_MapIdx_0__Array_mapFinIdxM_map_match__1_splitter(lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t lean_nat_dec_eq(lean_object*, lean_object*); +lean_object* lean_nat_sub(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Array_MapIdx_0__Array_mapFinIdxM_map_match__1_splitter___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Array_MapIdx_0__Array_mapFinIdxM_map_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; uint8_t x_6; +x_5 = lean_unsigned_to_nat(0u); +x_6 = lean_nat_dec_eq(x_1, x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_dec(x_3); +x_7 = lean_unsigned_to_nat(1u); +x_8 = lean_nat_sub(x_1, x_7); +x_9 = lean_apply_2(x_4, x_8, lean_box(0)); +return x_9; +} +else +{ +lean_object* x_10; +lean_dec(x_4); +x_10 = lean_apply_1(x_3, lean_box(0)); +return x_10; +} +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Array_MapIdx_0__Array_mapFinIdxM_map_match__1_splitter(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = lean_alloc_closure((void*)(l___private_Init_Data_Array_MapIdx_0__Array_mapFinIdxM_map_match__1_splitter___rarg___boxed), 4, 0); +return x_5; +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Array_MapIdx_0__Array_mapFinIdxM_map_match__1_splitter___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l___private_Init_Data_Array_MapIdx_0__Array_mapFinIdxM_map_match__1_splitter___rarg(x_1, x_2, x_3, x_4); +lean_dec(x_1); +return x_5; +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Array_MapIdx_0__Array_mapFinIdxM_map_match__1_splitter___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l___private_Init_Data_Array_MapIdx_0__Array_mapFinIdxM_map_match__1_splitter(x_1, x_2, x_3, x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_5; +} +} +lean_object* initialize_Init_Data_Array_Lemmas(uint8_t builtin, lean_object*); +lean_object* initialize_Init_Data_List_MapIdx(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Init_Data_Array_MapIdx(uint8_t builtin, lean_object* w) { +lean_object * res; +if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); +_G_initialized = true; +res = initialize_Init_Data_Array_Lemmas(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Init_Data_List_MapIdx(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +return lean_io_result_mk_ok(lean_box(0)); +} +#ifdef __cplusplus +} +#endif diff --git a/stage0/stdlib/Init/Data/Array/Mem.c b/stage0/stdlib/Init/Data/Array/Mem.c index 2f17a80f5976..c7145d3bb814 100644 --- a/stage0/stdlib/Init/Data/Array/Mem.c +++ b/stage0/stdlib/Init/Data/Array/Mem.c @@ -40,7 +40,6 @@ uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__11; static lean_object* l_Array_tacticArray__get__dec___closed__4; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__28; -LEAN_EXPORT lean_object* l_Array_instMembership(lean_object*); static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__40; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__27; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__1; @@ -128,14 +127,6 @@ LEAN_EXPORT lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__ lean_object* l_String_toSubstring_x27(lean_object*); static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__get__dec__1___closed__2; static lean_object* l_Array___aux__Init__Data__Array__Mem______macroRules__Array__tacticArray__mem__dec__1___closed__21; -LEAN_EXPORT lean_object* l_Array_instMembership(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_box(0); -return x_2; -} -} static lean_object* _init_l_Array_tacticArray__get__dec___closed__1() { _start: { diff --git a/stage0/stdlib/Init/Data/Hashable.c b/stage0/stdlib/Init/Data/Hashable.c index b212dceca9e0..2387afa1676f 100644 --- a/stage0/stdlib/Init/Data/Hashable.c +++ b/stage0/stdlib/Init/Data/Hashable.c @@ -20,6 +20,7 @@ uint64_t lean_uint64_of_nat(lean_object*); uint64_t lean_uint64_mix_hash(uint64_t, uint64_t); LEAN_EXPORT lean_object* l_instHashableProd(lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); +LEAN_EXPORT lean_object* l_instHashableChar___boxed(lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at_instHashableList___spec__1(lean_object*); LEAN_EXPORT lean_object* l_hash64___boxed(lean_object*); LEAN_EXPORT lean_object* l_instHashableInt___boxed(lean_object*); @@ -57,6 +58,7 @@ LEAN_EXPORT lean_object* l_instHashable___boxed(lean_object*, lean_object*); uint8_t lean_int_dec_lt(lean_object*, lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); lean_object* lean_nat_mul(lean_object*, lean_object*); +LEAN_EXPORT uint64_t l_instHashableChar(uint32_t); LEAN_EXPORT lean_object* l_instHashableOption(lean_object*); LEAN_EXPORT uint64_t l_hash64(uint64_t); static lean_object* l_instHashableInt___closed__1; @@ -524,6 +526,25 @@ lean_dec(x_1); return x_2; } } +LEAN_EXPORT uint64_t l_instHashableChar(uint32_t x_1) { +_start: +{ +uint64_t x_2; +x_2 = lean_uint32_to_uint64(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_instHashableChar___boxed(lean_object* x_1) { +_start: +{ +uint32_t x_2; uint64_t x_3; lean_object* x_4; +x_2 = lean_unbox_uint32(x_1); +lean_dec(x_1); +x_3 = l_instHashableChar(x_2); +x_4 = lean_box_uint64(x_3); +return x_4; +} +} static lean_object* _init_l_instHashableInt___closed__1() { _start: { diff --git a/stage0/stdlib/Init/Data/List/Basic.c b/stage0/stdlib/Init/Data/List/Basic.c index 46a7d0004e88..e228f45a6172 100644 --- a/stage0/stdlib/Init/Data/List/Basic.c +++ b/stage0/stdlib/Init/Data/List/Basic.c @@ -44,7 +44,7 @@ LEAN_EXPORT lean_object* l_List_enum___rarg(lean_object*); LEAN_EXPORT lean_object* l_List_join(lean_object*); LEAN_EXPORT lean_object* l_List_min_x3f(lean_object*); LEAN_EXPORT lean_object* l_List_zipWith(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_pure(lean_object*); +LEAN_EXPORT lean_object* l_List_pure(lean_object*, lean_object*); static lean_object* l_List___aux__Init__Data__List__Basic______macroRules__List__term___x3c_x3a_x2b____1___closed__4; LEAN_EXPORT lean_object* l_List_mapTR_loop(lean_object*, lean_object*); static lean_object* l_List___aux__Init__Data__List__Basic______macroRules__List__term___x3c_x2b____1___closed__1; @@ -94,6 +94,7 @@ static lean_object* l_List_term___x3c_x2b_x3a_____closed__4; LEAN_EXPORT lean_object* l_List_head_x3f___rarg___boxed(lean_object*); LEAN_EXPORT lean_object* l_List_countP_go___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_List___aux__Init__Data__List__Basic______macroRules__List__term___x7e____1___closed__6; +LEAN_EXPORT lean_object* l_List_modifyTailIdx___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Basic_0__List_flatten_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_term___x3c_x3a_x2b__; static lean_object* l_List___aux__Init__Data__List__Basic______macroRules__List__term___x3c_x3a_x2b____1___closed__2; @@ -109,6 +110,7 @@ static lean_object* l_List_term___x3c_x3a_x2b_x3a_____closed__2; LEAN_EXPORT lean_object* l_List_iotaTR_go(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_head_x3f___rarg(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Basic_0__List_range_x27TR_go_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_List_Basic_0__List_take_match__1_splitter(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_sum(lean_object*); LEAN_EXPORT lean_object* l_List_find_x3f___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_range_x27(lean_object*, lean_object*, lean_object*); @@ -120,6 +122,7 @@ static lean_object* l_List_term___x3c_x2b_____closed__9; static lean_object* l_List___aux__Init__Data__List__Basic______macroRules__List__term___x7e____1___closed__4; LEAN_EXPORT lean_object* l_List_instHasSubset(lean_object*); uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_flatMap___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List___aux__Init__Data__List__Basic______unexpand__List__Perm__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_bind(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_find_x3f(lean_object*); @@ -141,6 +144,7 @@ LEAN_EXPORT lean_object* l_List_rightpad___rarg(lean_object*, lean_object*, lean LEAN_EXPORT lean_object* l_List_instEmptyCollection(lean_object*); LEAN_EXPORT lean_object* l_List_head___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_beq___rarg___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_modify(lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_term___x3c_x2b__; LEAN_EXPORT lean_object* l_List_getD(lean_object*); @@ -242,6 +246,7 @@ LEAN_EXPORT lean_object* l_List_erase___rarg(lean_object*, lean_object*, lean_ob LEAN_EXPORT lean_object* l_List_indexOf___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_splitAt_go___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldr___at_Nat_sum___spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_List_Basic_0__List_take_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_eraseDups___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_replicateTR___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_enumFrom(lean_object*); @@ -260,6 +265,7 @@ LEAN_EXPORT lean_object* l_List_lookup___rarg(lean_object*, lean_object*, lean_o LEAN_EXPORT lean_object* l_List_headD(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Basic_0__List_beq_match__1_splitter(lean_object*, lean_object*); lean_object* l_List_lengthTRAux___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_modifyHead___rarg(lean_object*, lean_object*); lean_object* l_Lean_addMacroScope(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Basic_0__List_mapTR_loop_match__1_splitter(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_isPerm(lean_object*); @@ -267,12 +273,14 @@ LEAN_EXPORT lean_object* l_List_instDecidableRelSubsetOfDecidableEq(lean_object* LEAN_EXPORT lean_object* l_List_removeAll___rarg(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l_List___aux__Init__Data__List__Basic______macroRules__List__term___x3c_x2b____1___closed__6; +LEAN_EXPORT lean_object* l_List_singleton(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Basic_0__List_replicateTR_loop_match__1_splitter(lean_object*, lean_object*); lean_object* l_Lean_Syntax_node2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_unzip(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Basic_0__List_length_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_count(lean_object*); lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_modify___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_List___aux__Init__Data__List__Basic______macroRules__List__term___x7e____1___closed__2; LEAN_EXPORT lean_object* l_List_erase(lean_object*); LEAN_EXPORT lean_object* l_List_findIdx_go___at_List_indexOf___spec__1(lean_object*); @@ -326,6 +334,7 @@ static lean_object* l_List___aux__Init__Data__List__Basic______macroRules__List_ LEAN_EXPORT lean_object* l_List___aux__Init__Data__List__Basic______macroRules__List__term___x3c_x2b____1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_instLEOfLT___boxed(lean_object*, lean_object*); static lean_object* l_List_term___x3c_x2b_____closed__11; +LEAN_EXPORT lean_object* l_List_singleton___rarg(lean_object*); static lean_object* l_List_term___x3c_x3a_x2b_____closed__2; LEAN_EXPORT lean_object* l_List___aux__Init__Data__List__Basic______macroRules__List__term___x3c_x3a_x2b____1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_tail_x3f___rarg(lean_object*); @@ -335,6 +344,7 @@ LEAN_EXPORT lean_object* l_List_getLast_x3f___rarg(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Basic_0__List_dropLast_match__1_splitter(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_countP_go___at_List_count___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_term___x3c_x2b_____closed__8; +LEAN_EXPORT lean_object* l_List_modify___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_decidableBAll___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_tailD___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_findIdx(lean_object*); @@ -387,6 +397,7 @@ LEAN_EXPORT lean_object* l_List_splitAt_go(lean_object*); static lean_object* l_List_term___x3c_x3a_x2b_x3a_____closed__3; LEAN_EXPORT lean_object* l_List_get_x3f(lean_object*); LEAN_EXPORT lean_object* l_List_beq(lean_object*); +LEAN_EXPORT lean_object* l_List_modifyHead(lean_object*); LEAN_EXPORT lean_object* l_List___aux__Init__Data__List__Basic______unexpand__List__IsPrefix__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_intersperse___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_leftpad___rarg(lean_object*, lean_object*, lean_object*); @@ -401,6 +412,7 @@ LEAN_EXPORT lean_object* l_List_intersperseTR___rarg(lean_object*, lean_object*) lean_object* lean_nat_mul(lean_object*, lean_object*); static lean_object* l_List___aux__Init__Data__List__Basic______macroRules__List__term___x3c_x2b____1___closed__8; LEAN_EXPORT lean_object* l_List_leftpadTR___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_modifyTailIdx(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Basic_0__List_replicateTR_loop_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_term___x7e_____closed__5; LEAN_EXPORT lean_object* l_List_nodupDecidable___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); @@ -427,10 +439,11 @@ LEAN_EXPORT lean_object* l_List___aux__Init__Data__List__Basic______macroRules__ LEAN_EXPORT lean_object* l_List___aux__Init__Data__List__Basic______unexpand__List__Sublist__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_dropWhile___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_instDecidableMemOfLawfulBEq(lean_object*); -LEAN_EXPORT lean_object* l_List_pure___rarg(lean_object*); +LEAN_EXPORT lean_object* l_List_pure___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR(lean_object*, lean_object*); static lean_object* l_List___aux__Init__Data__List__Basic______macroRules__List__term___x3c_x3a_x2b_x3a____1___closed__4; static lean_object* l_List_term___x3c_x3a_x2b_____closed__4; +LEAN_EXPORT lean_object* l___private_Init_Data_List_Basic_0__List_take_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List___aux__Init__Data__List__Basic______macroRules__List__term___x3c_x2b____1___closed__7; LEAN_EXPORT lean_object* l_List_minimum_x3f(lean_object*); LEAN_EXPORT lean_object* l_List_append___rarg___boxed(lean_object*, lean_object*); @@ -467,6 +480,7 @@ LEAN_EXPORT lean_object* l_List_replicateTR_loop(lean_object*); static lean_object* l_List_instAppend___closed__1; LEAN_EXPORT lean_object* l_List_getLastD___rarg___boxed(lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_modifyTailIdx___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_insert(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Basic_0__List_getLast_x3f_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_partition(lean_object*); @@ -474,6 +488,7 @@ LEAN_EXPORT lean_object* l___private_Init_Data_List_Basic_0__List_beq_match__1_s LEAN_EXPORT lean_object* l_List_map___at_List_zipWithAll___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Basic_0__List_iotaTR_go_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_flatMap(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldr___at_List_sum___spec__1(lean_object*); LEAN_EXPORT lean_object* l_List_unzipTR(lean_object*, lean_object*); static lean_object* l_List_term___x3c_x2b_____closed__6; @@ -1936,7 +1951,7 @@ x_2 = lean_alloc_closure((void*)(l_List_join___rarg), 1, 0); return x_2; } } -LEAN_EXPORT lean_object* l_List_pure___rarg(lean_object* x_1) { +LEAN_EXPORT lean_object* l_List_singleton___rarg(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; @@ -1947,15 +1962,31 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_List_pure(lean_object* x_1) { +LEAN_EXPORT lean_object* l_List_singleton(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_List_pure___rarg), 1, 0); +x_2 = lean_alloc_closure((void*)(l_List_singleton___rarg), 1, 0); return x_2; } } -LEAN_EXPORT lean_object* l_List_bind___rarg(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_pure___rarg(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_apply_1(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_List_pure(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_List_pure___rarg), 2, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_List_flatMap___rarg(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; lean_object* x_4; @@ -1964,11 +1995,11 @@ x_4 = l_List_flatten___rarg(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_List_bind(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMap(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_List_bind___rarg), 2, 0); +x_3 = lean_alloc_closure((void*)(l_List_flatMap___rarg), 2, 0); return x_3; } } @@ -2011,6 +2042,23 @@ lean_dec(x_2); return x_4; } } +LEAN_EXPORT lean_object* l_List_bind___rarg(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; +x_3 = l_List_map___rarg(x_2, x_1); +x_4 = l_List_flatten___rarg(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l_List_bind(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_List_bind___rarg), 2, 0); +return x_3; +} +} LEAN_EXPORT lean_object* l_List_replicate___rarg(lean_object* x_1, lean_object* x_2) { _start: { @@ -5303,6 +5351,213 @@ x_2 = lean_alloc_closure((void*)(l_List_insert___rarg), 3, 0); return x_2; } } +LEAN_EXPORT lean_object* l_List_modifyTailIdx___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; uint8_t x_5; +x_4 = lean_unsigned_to_nat(0u); +x_5 = lean_nat_dec_eq(x_2, x_4); +if (x_5 == 0) +{ +if (lean_obj_tag(x_3) == 0) +{ +lean_object* x_6; +lean_dec(x_1); +x_6 = lean_box(0); +return x_6; +} +else +{ +uint8_t x_7; +x_7 = !lean_is_exclusive(x_3); +if (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_3, 1); +x_9 = lean_unsigned_to_nat(1u); +x_10 = lean_nat_sub(x_2, x_9); +x_11 = l_List_modifyTailIdx___rarg(x_1, x_10, x_8); +lean_dec(x_10); +lean_ctor_set(x_3, 1, x_11); +return x_3; +} +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; +x_12 = lean_ctor_get(x_3, 0); +x_13 = lean_ctor_get(x_3, 1); +lean_inc(x_13); +lean_inc(x_12); +lean_dec(x_3); +x_14 = lean_unsigned_to_nat(1u); +x_15 = lean_nat_sub(x_2, x_14); +x_16 = l_List_modifyTailIdx___rarg(x_1, x_15, x_13); +lean_dec(x_15); +x_17 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_17, 0, x_12); +lean_ctor_set(x_17, 1, x_16); +return x_17; +} +} +} +else +{ +lean_object* x_18; +x_18 = lean_apply_1(x_1, x_3); +return x_18; +} +} +} +LEAN_EXPORT lean_object* l_List_modifyTailIdx(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_List_modifyTailIdx___rarg___boxed), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_List_modifyTailIdx___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_List_modifyTailIdx___rarg(x_1, x_2, x_3); +lean_dec(x_2); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_List_Basic_0__List_take_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; uint8_t x_7; +x_6 = lean_unsigned_to_nat(0u); +x_7 = lean_nat_dec_eq(x_1, x_6); +if (x_7 == 0) +{ +lean_object* x_8; lean_object* x_9; +lean_dec(x_3); +x_8 = lean_unsigned_to_nat(1u); +x_9 = lean_nat_sub(x_1, x_8); +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_10; +lean_dec(x_5); +x_10 = lean_apply_1(x_4, x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; +lean_dec(x_4); +x_11 = lean_ctor_get(x_2, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_2, 1); +lean_inc(x_12); +lean_dec(x_2); +x_13 = lean_apply_3(x_5, x_9, x_11, x_12); +return x_13; +} +} +else +{ +lean_object* x_14; +lean_dec(x_5); +lean_dec(x_4); +x_14 = lean_apply_1(x_3, x_2); +return x_14; +} +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_List_Basic_0__List_take_match__1_splitter(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l___private_Init_Data_List_Basic_0__List_take_match__1_splitter___rarg___boxed), 5, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_List_Basic_0__List_take_match__1_splitter___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; +x_6 = l___private_Init_Data_List_Basic_0__List_take_match__1_splitter___rarg(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_1); +return x_6; +} +} +LEAN_EXPORT lean_object* l_List_modifyHead___rarg(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_3; +lean_dec(x_1); +x_3 = lean_box(0); +return x_3; +} +else +{ +uint8_t x_4; +x_4 = !lean_is_exclusive(x_2); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; +x_5 = lean_ctor_get(x_2, 0); +x_6 = lean_apply_1(x_1, x_5); +lean_ctor_set(x_2, 0, x_6); +return x_2; +} +else +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_7 = lean_ctor_get(x_2, 0); +x_8 = lean_ctor_get(x_2, 1); +lean_inc(x_8); +lean_inc(x_7); +lean_dec(x_2); +x_9 = lean_apply_1(x_1, x_7); +x_10 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set(x_10, 1, x_8); +return x_10; +} +} +} +} +LEAN_EXPORT lean_object* l_List_modifyHead(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_List_modifyHead___rarg), 2, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_List_modify___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; +x_4 = lean_alloc_closure((void*)(l_List_modifyHead___rarg), 2, 1); +lean_closure_set(x_4, 0, x_1); +x_5 = l_List_modifyTailIdx___rarg(x_4, x_2, x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_List_modify(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_List_modify___rarg___boxed), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_List_modify___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_List_modify___rarg(x_1, x_2, x_3); +lean_dec(x_2); +return x_4; +} +} LEAN_EXPORT lean_object* l_List_erase___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { diff --git a/stage0/stdlib/Init/Data/List/Impl.c b/stage0/stdlib/Init/Data/List/Impl.c index a0928ff7ead1..30e6ca65356c 100644 --- a/stage0/stdlib/Init/Data/List/Impl.c +++ b/stage0/stdlib/Init/Data/List/Impl.c @@ -14,16 +14,19 @@ extern "C" { #endif LEAN_EXPORT lean_object* l_List_zipWithTR(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_modifyTR_go___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_filter_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_intercalateTR_go___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_setTR_go___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_enumFromTR___spec__2(lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_modifyTR_go___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_enumFromTR___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_eraseIdxTR_go___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_List_bindTR___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_modifyTR_go___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_setTR_go___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_eraseTR(lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_eraseIdxTR_go___spec__2___rarg(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_modifyTR_go___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_zipWithTR_go_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_takeTR___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_eraseTR_go___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); @@ -37,6 +40,7 @@ LEAN_EXPORT lean_object* l_List_erasePTR___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_eraseIdx_match__1_splitter(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_zipWithTR_go___rarg(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); +LEAN_EXPORT lean_object* l_List_flatMapTR_go(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_enumFromTR(lean_object*); LEAN_EXPORT lean_object* l_List_takeTR_go___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterMapTR_go(lean_object*, lean_object*); @@ -44,7 +48,6 @@ LEAN_EXPORT lean_object* l_List_replaceTR_go___rarg(lean_object*, lean_object*, LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_intercalateTR_match__1_splitter(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_setTR_go(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_setTR_go_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_bindTR_go___at_List_flattenTR___spec__1___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_intercalateTR_go___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_takeWhileTR___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_eraseTR_go___spec__2___rarg(lean_object*, size_t, size_t, lean_object*); @@ -52,7 +55,6 @@ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_enumFromTR___spec__ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_intercalateTR_go___spec__2___rarg(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_List_takeTR(lean_object*); LEAN_EXPORT lean_object* l_List_eraseTR_go(lean_object*); -LEAN_EXPORT lean_object* l_List_bindTR(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_setTR_go___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_setTR_go___spec__2___rarg(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_List_replaceTR(lean_object*); @@ -60,13 +62,13 @@ LEAN_EXPORT lean_object* l_List_dropLastTR___rarg(lean_object*); size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_List_intercalateTR(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_filterMapTR_go_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_bindTR_go___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_modifyTR_go___spec__2(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_intercalateTR_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterMapTR(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_eraseTR_go___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_intercalateTR_go_match__1_splitter(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_modifyTR_go(lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_intercalateTR_go___spec__2(lean_object*); -LEAN_EXPORT lean_object* l_List_bindTR_go(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_eraseTR_go___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_enumFromTR___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); lean_object* lean_array_pop(lean_object*); @@ -75,7 +77,6 @@ lean_object* lean_array_to_list(lean_object*); LEAN_EXPORT lean_object* l_List_foldrTR(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_setTR_go___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_eraseIdxTR_go(lean_object*); -LEAN_EXPORT lean_object* l_List_bindTR_go___at_List_flattenTR___spec__1(lean_object*); LEAN_EXPORT lean_object* l_List_flattenTR(lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_intercalateTR_go___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_filterMap_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); @@ -84,13 +85,16 @@ LEAN_EXPORT lean_object* l_List_eraseIdxTR(lean_object*); LEAN_EXPORT lean_object* l_List_erasePTR(lean_object*); LEAN_EXPORT lean_object* l_List_filterMapTR_go___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_enumFromTR___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_flatMapTR(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_enumFromTR___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_filter_match__1_splitter___rarg(uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_eraseIdxTR_go___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_intercalateTR_go(lean_object*); +LEAN_EXPORT lean_object* l_List_modifyTR(lean_object*); LEAN_EXPORT lean_object* l_List_takeWhileTR(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_filterMapTR_go_match__2_splitter(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_setTR_go_match__1_splitter(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_modifyTR___rarg(lean_object*, lean_object*, lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_enumFromTR___spec__1(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_replace_match__1_splitter(lean_object*, lean_object*); @@ -98,6 +102,7 @@ LEAN_EXPORT lean_object* l_List_erasePTR_go(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_intercalateTR_go_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_takeTR_go(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_takeWhileTR_go_match__1_splitter(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_flatMapTR_go___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_eraseTR_go___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_enumFromTR___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_eraseTR_go___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -110,6 +115,7 @@ LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_filterMapTR_go_ LEAN_EXPORT lean_object* l_List_zipWithTR_go(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterMapTR___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_replace_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at_List_flattenTR___spec__1___rarg(lean_object*, lean_object*); extern lean_object* l_Id_instMonad; LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_filterMapTR_go_match__1_splitter(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_flattenTR___rarg(lean_object*); @@ -134,7 +140,10 @@ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_intercalateTR_go___ LEAN_EXPORT lean_object* l_List_eraseIdxTR_go___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_eraseIdxTR_go___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_takeWhileTR_go(lean_object*); +LEAN_EXPORT lean_object* l_List_modifyTR_go___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_getLast_x3f_match__1_splitter(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_flatMapTR___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at_List_flattenTR___spec__1(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_zipWithTR_go_match__1_splitter(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_filter_match__1_splitter(lean_object*); @@ -145,6 +154,7 @@ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_intercalateTR_go___ LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_enumFrom_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_setTR___rarg___closed__1; LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_setTR_go___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_modifyTR_go___spec__2___rarg(lean_object*, size_t, size_t, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_getLast_x3f_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_eraseIdx_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -715,7 +725,7 @@ x_3 = lean_alloc_closure((void*)(l_List_foldrTR___rarg), 3, 0); return x_3; } } -LEAN_EXPORT lean_object* l_List_bindTR_go___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_2) == 0) @@ -742,32 +752,32 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_List_bindTR_go(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_List_bindTR_go___rarg), 3, 0); +x_3 = lean_alloc_closure((void*)(l_List_flatMapTR_go___rarg), 3, 0); return x_3; } } -LEAN_EXPORT lean_object* l_List_bindTR___rarg(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMapTR___rarg(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; lean_object* x_4; x_3 = l_List_setTR___rarg___closed__1; -x_4 = l_List_bindTR_go___rarg(x_2, x_1, x_3); +x_4 = l_List_flatMapTR_go___rarg(x_2, x_1, x_3); return x_4; } } -LEAN_EXPORT lean_object* l_List_bindTR(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMapTR(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_List_bindTR___rarg), 2, 0); +x_3 = lean_alloc_closure((void*)(l_List_flatMapTR___rarg), 2, 0); return x_3; } } -LEAN_EXPORT lean_object* l_List_bindTR_go___at_List_flattenTR___spec__1___rarg(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at_List_flattenTR___spec__1___rarg(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -791,11 +801,11 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_List_bindTR_go___at_List_flattenTR___spec__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at_List_flattenTR___spec__1(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_List_bindTR_go___at_List_flattenTR___spec__1___rarg), 2, 0); +x_2 = lean_alloc_closure((void*)(l_List_flatMapTR_go___at_List_flattenTR___spec__1___rarg), 2, 0); return x_2; } } @@ -804,7 +814,7 @@ LEAN_EXPORT lean_object* l_List_flattenTR___rarg(lean_object* x_1) { { lean_object* x_2; lean_object* x_3; x_2 = l_List_setTR___rarg___closed__1; -x_3 = l_List_bindTR_go___at_List_flattenTR___spec__1___rarg(x_1, x_2); +x_3 = l_List_flatMapTR_go___at_List_flattenTR___spec__1___rarg(x_1, x_2); return x_3; } } @@ -1267,6 +1277,287 @@ x_3 = lean_alloc_closure((void*)(l___private_Init_Data_List_Impl_0__List_replace return x_3; } } +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_modifyTR_go___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_eq(x_2, x_3); +if (x_5 == 0) +{ +size_t x_6; size_t x_7; lean_object* x_8; lean_object* x_9; +x_6 = 1; +x_7 = lean_usize_sub(x_2, x_6); +x_8 = lean_array_uget(x_1, x_7); +x_9 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_9, 0, x_8); +lean_ctor_set(x_9, 1, x_4); +x_2 = x_7; +x_4 = x_9; +goto _start; +} +else +{ +return x_4; +} +} +} +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_modifyTR_go___spec__1(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_List_modifyTR_go___spec__1___rarg___boxed), 4, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_modifyTR_go___spec__2___rarg(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; +x_5 = lean_usize_dec_eq(x_2, x_3); +if (x_5 == 0) +{ +size_t x_6; size_t x_7; lean_object* x_8; lean_object* x_9; +x_6 = 1; +x_7 = lean_usize_sub(x_2, x_6); +x_8 = lean_array_uget(x_1, x_7); +x_9 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_9, 0, x_8); +lean_ctor_set(x_9, 1, x_4); +x_2 = x_7; +x_4 = x_9; +goto _start; +} +else +{ +return x_4; +} +} +} +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_modifyTR_go___spec__2(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_List_modifyTR_go___spec__2___rarg___boxed), 4, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_List_modifyTR_go___rarg(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_dec(x_3); +lean_dec(x_1); +x_5 = lean_array_to_list(x_4); +return x_5; +} +else +{ +uint8_t x_6; +x_6 = !lean_is_exclusive(x_2); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; +x_7 = lean_ctor_get(x_2, 0); +x_8 = lean_ctor_get(x_2, 1); +x_9 = lean_unsigned_to_nat(0u); +x_10 = lean_nat_dec_eq(x_3, x_9); +if (x_10 == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; +lean_free_object(x_2); +x_11 = lean_unsigned_to_nat(1u); +x_12 = lean_nat_sub(x_3, x_11); +lean_dec(x_3); +x_13 = lean_array_push(x_4, x_7); +x_2 = x_8; +x_3 = x_12; +x_4 = x_13; +goto _start; +} +else +{ +lean_object* x_15; lean_object* x_16; uint8_t x_17; +lean_dec(x_3); +x_15 = lean_apply_1(x_1, x_7); +lean_ctor_set(x_2, 0, x_15); +x_16 = lean_array_get_size(x_4); +x_17 = lean_nat_dec_le(x_16, x_16); +if (x_17 == 0) +{ +uint8_t x_18; +x_18 = lean_nat_dec_lt(x_9, x_16); +if (x_18 == 0) +{ +lean_dec(x_16); +lean_dec(x_4); +return x_2; +} +else +{ +size_t x_19; size_t x_20; lean_object* x_21; +x_19 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_20 = 0; +x_21 = l_Array_foldrMUnsafe_fold___at_List_modifyTR_go___spec__1___rarg(x_4, x_19, x_20, x_2); +lean_dec(x_4); +return x_21; +} +} +else +{ +uint8_t x_22; +x_22 = lean_nat_dec_lt(x_9, x_16); +if (x_22 == 0) +{ +lean_dec(x_16); +lean_dec(x_4); +return x_2; +} +else +{ +size_t x_23; size_t x_24; lean_object* x_25; +x_23 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_24 = 0; +x_25 = l_Array_foldrMUnsafe_fold___at_List_modifyTR_go___spec__2___rarg(x_4, x_23, x_24, x_2); +lean_dec(x_4); +return x_25; +} +} +} +} +else +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; +x_26 = lean_ctor_get(x_2, 0); +x_27 = lean_ctor_get(x_2, 1); +lean_inc(x_27); +lean_inc(x_26); +lean_dec(x_2); +x_28 = lean_unsigned_to_nat(0u); +x_29 = lean_nat_dec_eq(x_3, x_28); +if (x_29 == 0) +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_unsigned_to_nat(1u); +x_31 = lean_nat_sub(x_3, x_30); +lean_dec(x_3); +x_32 = lean_array_push(x_4, x_26); +x_2 = x_27; +x_3 = x_31; +x_4 = x_32; +goto _start; +} +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; +lean_dec(x_3); +x_34 = lean_apply_1(x_1, x_26); +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_34); +lean_ctor_set(x_35, 1, x_27); +x_36 = lean_array_get_size(x_4); +x_37 = lean_nat_dec_le(x_36, x_36); +if (x_37 == 0) +{ +uint8_t x_38; +x_38 = lean_nat_dec_lt(x_28, x_36); +if (x_38 == 0) +{ +lean_dec(x_36); +lean_dec(x_4); +return x_35; +} +else +{ +size_t x_39; size_t x_40; lean_object* x_41; +x_39 = lean_usize_of_nat(x_36); +lean_dec(x_36); +x_40 = 0; +x_41 = l_Array_foldrMUnsafe_fold___at_List_modifyTR_go___spec__1___rarg(x_4, x_39, x_40, x_35); +lean_dec(x_4); +return x_41; +} +} +else +{ +uint8_t x_42; +x_42 = lean_nat_dec_lt(x_28, x_36); +if (x_42 == 0) +{ +lean_dec(x_36); +lean_dec(x_4); +return x_35; +} +else +{ +size_t x_43; size_t x_44; lean_object* x_45; +x_43 = lean_usize_of_nat(x_36); +lean_dec(x_36); +x_44 = 0; +x_45 = l_Array_foldrMUnsafe_fold___at_List_modifyTR_go___spec__2___rarg(x_4, x_43, x_44, x_35); +lean_dec(x_4); +return x_45; +} +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_List_modifyTR_go(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_List_modifyTR_go___rarg), 4, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_modifyTR_go___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_foldrMUnsafe_fold___at_List_modifyTR_go___spec__1___rarg(x_1, x_5, x_6, x_4); +lean_dec(x_1); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_modifyTR_go___spec__2___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_foldrMUnsafe_fold___at_List_modifyTR_go___spec__2___rarg(x_1, x_5, x_6, x_4); +lean_dec(x_1); +return x_7; +} +} +LEAN_EXPORT lean_object* l_List_modifyTR___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; +x_4 = l_List_setTR___rarg___closed__1; +x_5 = l_List_modifyTR_go___rarg(x_1, x_3, x_2, x_4); +return x_5; +} +} +LEAN_EXPORT lean_object* l_List_modifyTR(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_List_modifyTR___rarg), 3, 0); +return x_2; +} +} LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_eraseTR_go___spec__1___rarg(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { diff --git a/stage0/stdlib/Init/Data/List/Monadic.c b/stage0/stdlib/Init/Data/List/Monadic.c index e7e783ea6c59..9f555f7dfdf5 100644 --- a/stage0/stdlib/Init/Data/List/Monadic.c +++ b/stage0/stdlib/Init/Data/List/Monadic.c @@ -18,13 +18,17 @@ LEAN_EXPORT lean_object* l___private_Init_Data_List_Monadic_0__List_mapM_loop_ma LEAN_EXPORT lean_object* l_List_mapM_x27___rarg___lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapM_x27(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Monadic_0__List_anyM_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_List_Monadic_0__List_forIn_loop_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_List_Monadic_0__List_forIn_loop_match__1_splitter(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Monadic_0__List_mapM_x27_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Monadic_0__List_findM_x3f_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Monadic_0__List_anyM_match__1_splitter___rarg(uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Monadic_0__List_anyM_match__1_splitter(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Monadic_0__List_mapA_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_List_Monadic_0__List_forIn_x27__cons_match__1_splitter(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapM_x27___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Monadic_0__List_mapA_match__1_splitter(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_List_Monadic_0__List_forIn_x27__cons_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Monadic_0__List_mapM_x27_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Monadic_0__List_mapA_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Monadic_0__List_filterAuxM_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*); @@ -292,6 +296,72 @@ lean_dec(x_2); return x_4; } } +LEAN_EXPORT lean_object* l___private_Init_Data_List_Monadic_0__List_forIn_loop_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_4; lean_object* x_5; +lean_dec(x_3); +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_apply_1(x_2, x_4); +return x_5; +} +else +{ +lean_object* x_6; lean_object* x_7; +lean_dec(x_2); +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +lean_dec(x_1); +x_7 = lean_apply_1(x_3, x_6); +return x_7; +} +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_List_Monadic_0__List_forIn_loop_match__1_splitter(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l___private_Init_Data_List_Monadic_0__List_forIn_loop_match__1_splitter___rarg), 3, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_List_Monadic_0__List_forIn_x27__cons_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_4; lean_object* x_5; +lean_dec(x_3); +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_apply_1(x_2, x_4); +return x_5; +} +else +{ +lean_object* x_6; lean_object* x_7; +lean_dec(x_2); +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +lean_dec(x_1); +x_7 = lean_apply_1(x_3, x_6); +return x_7; +} +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_List_Monadic_0__List_forIn_x27__cons_match__1_splitter(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l___private_Init_Data_List_Monadic_0__List_forIn_x27__cons_match__1_splitter___rarg), 3, 0); +return x_3; +} +} LEAN_EXPORT lean_object* l___private_Init_Data_List_Monadic_0__List_anyM_match__1_splitter___rarg(uint8_t x_1, lean_object* x_2, lean_object* x_3) { _start: { diff --git a/stage0/stdlib/Init/Data/List/Nat.c b/stage0/stdlib/Init/Data/List/Nat.c index c1510a26117e..9c058e6d0e11 100644 --- a/stage0/stdlib/Init/Data/List/Nat.c +++ b/stage0/stdlib/Init/Data/List/Nat.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Init.Data.List.Nat -// Imports: Init.Data.List.Nat.Basic Init.Data.List.Nat.Pairwise Init.Data.List.Nat.Range Init.Data.List.Nat.Sublist Init.Data.List.Nat.TakeDrop Init.Data.List.Nat.Count Init.Data.List.Nat.Erase Init.Data.List.Nat.Find +// Imports: Init.Data.List.Nat.Basic Init.Data.List.Nat.Pairwise Init.Data.List.Nat.Range Init.Data.List.Nat.Sublist Init.Data.List.Nat.TakeDrop Init.Data.List.Nat.Count Init.Data.List.Nat.Erase Init.Data.List.Nat.Find Init.Data.List.Nat.BEq Init.Data.List.Nat.Modify #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -21,6 +21,8 @@ lean_object* initialize_Init_Data_List_Nat_TakeDrop(uint8_t builtin, lean_object lean_object* initialize_Init_Data_List_Nat_Count(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_List_Nat_Erase(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_List_Nat_Find(uint8_t builtin, lean_object*); +lean_object* initialize_Init_Data_List_Nat_BEq(uint8_t builtin, lean_object*); +lean_object* initialize_Init_Data_List_Nat_Modify(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Init_Data_List_Nat(uint8_t builtin, lean_object* w) { lean_object * res; @@ -50,6 +52,12 @@ lean_dec_ref(res); res = initialize_Init_Data_List_Nat_Find(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +res = initialize_Init_Data_List_Nat_BEq(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Init_Data_List_Nat_Modify(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Init/Data/List/Nat/BEq.c b/stage0/stdlib/Init/Data/List/Nat/BEq.c new file mode 100644 index 000000000000..bc217a32439d --- /dev/null +++ b/stage0/stdlib/Init/Data/List/Nat/BEq.c @@ -0,0 +1,94 @@ +// Lean compiler output +// Module: Init.Data.List.Nat.BEq +// Imports: Init.Data.Nat.Lemmas Init.Data.List.Basic +#include +#if defined(__clang__) +#pragma clang diagnostic ignored "-Wunused-parameter" +#pragma clang diagnostic ignored "-Wunused-label" +#elif defined(__GNUC__) && !defined(__CLANG__) +#pragma GCC diagnostic ignored "-Wunused-parameter" +#pragma GCC diagnostic ignored "-Wunused-label" +#pragma GCC diagnostic ignored "-Wunused-but-set-variable" +#endif +#ifdef __cplusplus +extern "C" { +#endif +LEAN_EXPORT lean_object* l___private_Init_Data_List_Nat_BEq_0__List_isEqv_match__1_splitter(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_List_Nat_BEq_0__List_isEqv_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_List_Nat_BEq_0__List_isEqv_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_dec(x_5); +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_7; +lean_dec(x_6); +x_7 = lean_apply_1(x_4, x_3); +return x_7; +} +else +{ +lean_object* x_8; +lean_dec(x_4); +x_8 = lean_apply_5(x_6, x_1, x_2, x_3, lean_box(0), lean_box(0)); +return x_8; +} +} +else +{ +lean_dec(x_4); +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_9; +lean_dec(x_5); +x_9 = lean_apply_5(x_6, x_1, x_2, x_3, lean_box(0), lean_box(0)); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +lean_dec(x_6); +x_10 = lean_ctor_get(x_1, 0); +lean_inc(x_10); +x_11 = lean_ctor_get(x_1, 1); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_2, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_2, 1); +lean_inc(x_13); +lean_dec(x_2); +x_14 = lean_apply_5(x_5, x_10, x_11, x_12, x_13, x_3); +return x_14; +} +} +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_List_Nat_BEq_0__List_isEqv_match__1_splitter(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l___private_Init_Data_List_Nat_BEq_0__List_isEqv_match__1_splitter___rarg), 6, 0); +return x_3; +} +} +lean_object* initialize_Init_Data_Nat_Lemmas(uint8_t builtin, lean_object*); +lean_object* initialize_Init_Data_List_Basic(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Init_Data_List_Nat_BEq(uint8_t builtin, lean_object* w) { +lean_object * res; +if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); +_G_initialized = true; +res = initialize_Init_Data_Nat_Lemmas(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Init_Data_List_Basic(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +return lean_io_result_mk_ok(lean_box(0)); +} +#ifdef __cplusplus +} +#endif diff --git a/stage0/stdlib/Init/Data/List/Nat/Modify.c b/stage0/stdlib/Init/Data/List/Nat/Modify.c new file mode 100644 index 000000000000..62264bb41a30 --- /dev/null +++ b/stage0/stdlib/Init/Data/List/Nat/Modify.c @@ -0,0 +1,73 @@ +// Lean compiler output +// Module: Init.Data.List.Nat.Modify +// Imports: Init.Data.List.Nat.TakeDrop Init.Data.List.Nat.Erase +#include +#if defined(__clang__) +#pragma clang diagnostic ignored "-Wunused-parameter" +#pragma clang diagnostic ignored "-Wunused-label" +#elif defined(__GNUC__) && !defined(__CLANG__) +#pragma GCC diagnostic ignored "-Wunused-parameter" +#pragma GCC diagnostic ignored "-Wunused-label" +#pragma GCC diagnostic ignored "-Wunused-but-set-variable" +#endif +#ifdef __cplusplus +extern "C" { +#endif +LEAN_EXPORT lean_object* l___private_Init_Data_List_Nat_Modify_0__Option_getD_match__1_splitter(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_List_Nat_Modify_0__Option_getD_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_List_Nat_Modify_0__Option_getD_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_List_Nat_Modify_0__Option_getD_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_dec(x_2); +lean_inc(x_3); +return x_3; +} +else +{ +lean_object* x_4; lean_object* x_5; +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_apply_1(x_2, x_4); +return x_5; +} +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_List_Nat_Modify_0__Option_getD_match__1_splitter(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l___private_Init_Data_List_Nat_Modify_0__Option_getD_match__1_splitter___rarg___boxed), 3, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_List_Nat_Modify_0__Option_getD_match__1_splitter___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Init_Data_List_Nat_Modify_0__Option_getD_match__1_splitter___rarg(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; +} +} +lean_object* initialize_Init_Data_List_Nat_TakeDrop(uint8_t builtin, lean_object*); +lean_object* initialize_Init_Data_List_Nat_Erase(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Init_Data_List_Nat_Modify(uint8_t builtin, lean_object* w) { +lean_object * res; +if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); +_G_initialized = true; +res = initialize_Init_Data_List_Nat_TakeDrop(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Init_Data_List_Nat_Erase(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +return lean_io_result_mk_ok(lean_box(0)); +} +#ifdef __cplusplus +} +#endif diff --git a/stage0/stdlib/Init/Data/Option/Basic.c b/stage0/stdlib/Init/Data/Option/Basic.c index ef68aa4ac0d5..f674f77fb5f5 100644 --- a/stage0/stdlib/Init/Data/Option/Basic.c +++ b/stage0/stdlib/Init/Data/Option/Basic.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Init.Data.Option.Basic -// Imports: Init.Core Init.Control.Basic Init.Coe +// Imports: Init.Control.Basic #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -2359,23 +2359,15 @@ lean_dec(x_2); return x_4; } } -lean_object* initialize_Init_Core(uint8_t builtin, lean_object*); lean_object* initialize_Init_Control_Basic(uint8_t builtin, lean_object*); -lean_object* initialize_Init_Coe(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Init_Data_Option_Basic(uint8_t builtin, lean_object* w) { lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init_Core(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Init_Control_Basic(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -res = initialize_Init_Coe(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); l_Option_toArray___rarg___closed__1 = _init_l_Option_toArray___rarg___closed__1(); lean_mark_persistent(l_Option_toArray___rarg___closed__1); l_Option_mapA___rarg___closed__1 = _init_l_Option_mapA___rarg___closed__1(); diff --git a/stage0/stdlib/Init/Data/Prod.c b/stage0/stdlib/Init/Data/Prod.c index fbc2f9481307..067ec63bf32c 100644 --- a/stage0/stdlib/Init/Data/Prod.c +++ b/stage0/stdlib/Init/Data/Prod.c @@ -13,6 +13,40 @@ #ifdef __cplusplus extern "C" { #endif +LEAN_EXPORT lean_object* l_Prod_swap___rarg___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Prod_swap___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Prod_swap(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Prod_swap___rarg(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_2 = lean_ctor_get(x_1, 1); +x_3 = lean_ctor_get(x_1, 0); +lean_inc(x_3); +lean_inc(x_2); +x_4 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_4, 0, x_2); +lean_ctor_set(x_4, 1, x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Prod_swap(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Prod_swap___rarg___boxed), 1, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Prod_swap___rarg___boxed(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = l_Prod_swap___rarg(x_1); +lean_dec(x_1); +return x_2; +} +} lean_object* initialize_Init_SimpLemmas(uint8_t builtin, lean_object*); lean_object* initialize_Init_NotationExtra(uint8_t builtin, lean_object*); static bool _G_initialized = false; diff --git a/stage0/stdlib/Init/Data/Repr.c b/stage0/stdlib/Init/Data/Repr.c index caf301c4dc36..ae1f05f84ab6 100644 --- a/stage0/stdlib/Init/Data/Repr.c +++ b/stage0/stdlib/Init/Data/Repr.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Init.Data.Repr -// Imports: Init.Data.Format.Basic Init.Data.Int.Basic Init.Data.Nat.Div Init.Data.UInt.BasicAux Init.Control.Id +// Imports: Init.Data.Format.Basic #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -4161,10 +4161,6 @@ return x_1; } } lean_object* initialize_Init_Data_Format_Basic(uint8_t builtin, lean_object*); -lean_object* initialize_Init_Data_Int_Basic(uint8_t builtin, lean_object*); -lean_object* initialize_Init_Data_Nat_Div(uint8_t builtin, lean_object*); -lean_object* initialize_Init_Data_UInt_BasicAux(uint8_t builtin, lean_object*); -lean_object* initialize_Init_Control_Id(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Init_Data_Repr(uint8_t builtin, lean_object* w) { lean_object * res; @@ -4173,18 +4169,6 @@ _G_initialized = true; res = initialize_Init_Data_Format_Basic(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -res = initialize_Init_Data_Int_Basic(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -res = initialize_Init_Data_Nat_Div(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -res = initialize_Init_Data_UInt_BasicAux(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -res = initialize_Init_Control_Id(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); l_instReprBool___closed__1 = _init_l_instReprBool___closed__1(); lean_mark_persistent(l_instReprBool___closed__1); l_instReprBool___closed__2 = _init_l_instReprBool___closed__2(); diff --git a/stage0/stdlib/Init/Data/SInt.c b/stage0/stdlib/Init/Data/SInt.c new file mode 100644 index 000000000000..ad16e914ae43 --- /dev/null +++ b/stage0/stdlib/Init/Data/SInt.c @@ -0,0 +1,29 @@ +// Lean compiler output +// Module: Init.Data.SInt +// Imports: Init.Data.SInt.Basic +#include +#if defined(__clang__) +#pragma clang diagnostic ignored "-Wunused-parameter" +#pragma clang diagnostic ignored "-Wunused-label" +#elif defined(__GNUC__) && !defined(__CLANG__) +#pragma GCC diagnostic ignored "-Wunused-parameter" +#pragma GCC diagnostic ignored "-Wunused-label" +#pragma GCC diagnostic ignored "-Wunused-but-set-variable" +#endif +#ifdef __cplusplus +extern "C" { +#endif +lean_object* initialize_Init_Data_SInt_Basic(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Init_Data_SInt(uint8_t builtin, lean_object* w) { +lean_object * res; +if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); +_G_initialized = true; +res = initialize_Init_Data_SInt_Basic(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +return lean_io_result_mk_ok(lean_box(0)); +} +#ifdef __cplusplus +} +#endif diff --git a/stage0/stdlib/Init/Data/SInt/Basic.c b/stage0/stdlib/Init/Data/SInt/Basic.c new file mode 100644 index 000000000000..c0c8607afb96 --- /dev/null +++ b/stage0/stdlib/Init/Data/SInt/Basic.c @@ -0,0 +1,912 @@ +// Lean compiler output +// Module: Init.Data.SInt.Basic +// Imports: Init.Data.UInt.Basic +#include +#if defined(__clang__) +#pragma clang diagnostic ignored "-Wunused-parameter" +#pragma clang diagnostic ignored "-Wunused-label" +#elif defined(__GNUC__) && !defined(__CLANG__) +#pragma GCC diagnostic ignored "-Wunused-parameter" +#pragma GCC diagnostic ignored "-Wunused-label" +#pragma GCC diagnostic ignored "-Wunused-but-set-variable" +#endif +#ifdef __cplusplus +extern "C" { +#endif +static lean_object* l_instModInt8___closed__1; +LEAN_EXPORT lean_object* l_instMulInt8; +LEAN_EXPORT lean_object* l_Int8_decLt___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_instDecidableLeInt8___boxed(lean_object*, lean_object*); +static lean_object* l_instDivInt8___closed__1; +LEAN_EXPORT lean_object* l_Int8_sub___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_instComplementInt8; +LEAN_EXPORT uint8_t l_instDecidableLtInt8(uint8_t, uint8_t); +LEAN_EXPORT lean_object* l_Int8_ofInt___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Int8_div___boxed(lean_object*, lean_object*); +uint8_t lean_int8_dec_eq(uint8_t, uint8_t); +LEAN_EXPORT lean_object* l_instSubInt8; +LEAN_EXPORT uint8_t l_instMaxInt8(uint8_t, uint8_t); +uint8_t lean_int8_shift_left(uint8_t, uint8_t); +LEAN_EXPORT uint8_t l_instInhabitedInt8; +static lean_object* l_instXorInt8___closed__1; +LEAN_EXPORT lean_object* l_Int8_toInt___boxed(lean_object*); +LEAN_EXPORT uint8_t l_instOfNatInt8(lean_object*); +LEAN_EXPORT lean_object* l_instOfNatInt8___boxed(lean_object*); +lean_object* lean_int8_to_int(uint8_t); +LEAN_EXPORT lean_object* l_instModInt8; +uint8_t lean_int8_mul(uint8_t, uint8_t); +uint8_t lean_int8_complement(uint8_t); +static uint8_t l_instInhabitedInt8___closed__1; +uint8_t lean_int8_div(uint8_t, uint8_t); +uint8_t lean_int8_mod(uint8_t, uint8_t); +uint8_t lean_int8_lor(uint8_t, uint8_t); +static lean_object* l_instToStringInt8___closed__1; +lean_object* lean_nat_to_int(lean_object*); +LEAN_EXPORT lean_object* l_Int8_decEq___boxed(lean_object*, lean_object*); +static lean_object* l_instMulInt8___closed__1; +uint8_t lean_int8_neg(uint8_t); +LEAN_EXPORT lean_object* l_Int8_lor___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_instDecidableLtInt8___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_instDecidableEqInt8___boxed(lean_object*, lean_object*); +lean_object* lean_uint8_to_nat(uint8_t); +LEAN_EXPORT lean_object* l_instDivInt8; +LEAN_EXPORT lean_object* l_instToStringInt8___boxed(lean_object*); +static lean_object* l_instNegInt8___closed__1; +uint8_t lean_int8_shift_right(uint8_t, uint8_t); +static lean_object* l_instAddInt8___closed__1; +LEAN_EXPORT lean_object* l_instOrOpInt8; +LEAN_EXPORT lean_object* l_Int8_size; +LEAN_EXPORT lean_object* l_instToStringInt8(uint8_t); +uint8_t lean_int8_sub(uint8_t, uint8_t); +LEAN_EXPORT lean_object* l_Int8_decLe___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_instAddInt8; +LEAN_EXPORT lean_object* l_Int8_toBitVec___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Int8_mod___boxed(lean_object*, lean_object*); +static lean_object* l_instSubInt8___closed__1; +LEAN_EXPORT uint8_t l_instDecidableEqInt8(uint8_t, uint8_t); +uint8_t lean_int8_add(uint8_t, uint8_t); +LEAN_EXPORT lean_object* l_Int8_ofNat___boxed(lean_object*); +static lean_object* l_instShiftRightInt8___closed__1; +LEAN_EXPORT lean_object* l_Int8_xor___boxed(lean_object*, lean_object*); +lean_object* lean_nat_abs(lean_object*); +LEAN_EXPORT lean_object* l_instNegInt8; +LEAN_EXPORT lean_object* l_Nat_toInt8___boxed(lean_object*); +uint8_t lean_int8_dec_lt(uint8_t, uint8_t); +LEAN_EXPORT lean_object* l_instLEInt8; +LEAN_EXPORT uint8_t l_Int_toInt8(lean_object*); +LEAN_EXPORT lean_object* l_Int8_toNat___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Int8_toBitVec(uint8_t); +LEAN_EXPORT lean_object* l_Int8_add___boxed(lean_object*, lean_object*); +static lean_object* l_instComplementInt8___closed__1; +LEAN_EXPORT lean_object* l_instXorInt8; +LEAN_EXPORT lean_object* l_Int8_shiftRight___boxed(lean_object*, lean_object*); +lean_object* l_Int_toNat(lean_object*); +LEAN_EXPORT lean_object* l_Int8_shiftLeft___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_instLTInt8; +uint8_t lean_int_dec_lt(lean_object*, lean_object*); +lean_object* lean_nat_sub(lean_object*, lean_object*); +static lean_object* l_instShiftLeftInt8___closed__1; +uint8_t lean_int8_of_int(lean_object*); +uint8_t lean_int8_dec_le(uint8_t, uint8_t); +uint8_t lean_int8_of_int(lean_object*); +LEAN_EXPORT uint8_t l_instDecidableLeInt8(uint8_t, uint8_t); +LEAN_EXPORT uint8_t l_instMinInt8(uint8_t, uint8_t); +LEAN_EXPORT lean_object* l_instMaxInt8___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_instShiftRightInt8; +LEAN_EXPORT lean_object* l_Int_toInt8___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Int8_complement___boxed(lean_object*); +lean_object* lean_string_append(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Int8_mul___boxed(lean_object*, lean_object*); +uint8_t lean_int8_xor(uint8_t, uint8_t); +LEAN_EXPORT lean_object* l_instMinInt8___boxed(lean_object*, lean_object*); +static lean_object* l_instOrOpInt8___closed__1; +LEAN_EXPORT lean_object* l_instAndOpInt8; +lean_object* lean_nat_add(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_instShiftLeftInt8; +static lean_object* l_instToStringInt8___closed__2; +LEAN_EXPORT uint8_t l_Nat_toInt8(lean_object*); +LEAN_EXPORT lean_object* l_Int8_neg___boxed(lean_object*); +lean_object* l___private_Init_Data_Repr_0__Nat_reprFast(lean_object*); +LEAN_EXPORT lean_object* l_Int8_land___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Int8_toNat(uint8_t); +uint8_t lean_int8_land(uint8_t, uint8_t); +static lean_object* l_instAndOpInt8___closed__1; +static lean_object* _init_l_Int8_size() { +_start: +{ +lean_object* x_1; +x_1 = lean_unsigned_to_nat(256u); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Int8_toBitVec(uint8_t x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_uint8_to_nat(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Int8_toBitVec___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_Int8_toBitVec(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Int8_ofInt___boxed(lean_object* x_1) { +_start: +{ +uint8_t x_2; lean_object* x_3; +x_2 = lean_int8_of_int(x_1); +lean_dec(x_1); +x_3 = lean_box(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Int8_ofNat___boxed(lean_object* x_1) { +_start: +{ +uint8_t x_2; lean_object* x_3; +x_2 = lean_int8_of_int(x_1); +lean_dec(x_1); +x_3 = lean_box(x_2); +return x_3; +} +} +LEAN_EXPORT uint8_t l_Int_toInt8(lean_object* x_1) { +_start: +{ +uint8_t x_2; +x_2 = lean_int8_of_int(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Int_toInt8___boxed(lean_object* x_1) { +_start: +{ +uint8_t x_2; lean_object* x_3; +x_2 = l_Int_toInt8(x_1); +lean_dec(x_1); +x_3 = lean_box(x_2); +return x_3; +} +} +LEAN_EXPORT uint8_t l_Nat_toInt8(lean_object* x_1) { +_start: +{ +uint8_t x_2; +x_2 = lean_int8_of_int(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Nat_toInt8___boxed(lean_object* x_1) { +_start: +{ +uint8_t x_2; lean_object* x_3; +x_2 = l_Nat_toInt8(x_1); +lean_dec(x_1); +x_3 = lean_box(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Int8_toInt___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 = lean_int8_to_int(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Int8_toNat(uint8_t x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; +x_2 = lean_int8_to_int(x_1); +x_3 = l_Int_toNat(x_2); +lean_dec(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Int8_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_Int8_toNat(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Int8_neg___boxed(lean_object* x_1) { +_start: +{ +uint8_t x_2; uint8_t x_3; lean_object* x_4; +x_2 = lean_unbox(x_1); +lean_dec(x_1); +x_3 = lean_int8_neg(x_2); +x_4 = lean_box(x_3); +return x_4; +} +} +static lean_object* _init_l_instToStringInt8___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(0u); +x_2 = lean_nat_to_int(x_1); +return x_2; +} +} +static lean_object* _init_l_instToStringInt8___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("-", 1, 1); +return x_1; +} +} +LEAN_EXPORT lean_object* l_instToStringInt8(uint8_t x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; uint8_t x_4; +x_2 = lean_int8_to_int(x_1); +x_3 = l_instToStringInt8___closed__1; +x_4 = lean_int_dec_lt(x_2, x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; +x_5 = lean_nat_abs(x_2); +lean_dec(x_2); +x_6 = l___private_Init_Data_Repr_0__Nat_reprFast(x_5); +return x_6; +} +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; +x_7 = lean_nat_abs(x_2); +lean_dec(x_2); +x_8 = lean_unsigned_to_nat(1u); +x_9 = lean_nat_sub(x_7, x_8); +lean_dec(x_7); +x_10 = lean_nat_add(x_9, x_8); +lean_dec(x_9); +x_11 = l___private_Init_Data_Repr_0__Nat_reprFast(x_10); +x_12 = l_instToStringInt8___closed__2; +x_13 = lean_string_append(x_12, x_11); +lean_dec(x_11); +return x_13; +} +} +} +LEAN_EXPORT lean_object* l_instToStringInt8___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_instToStringInt8(x_2); +return x_3; +} +} +LEAN_EXPORT uint8_t l_instOfNatInt8(lean_object* x_1) { +_start: +{ +uint8_t x_2; +x_2 = lean_int8_of_int(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_instOfNatInt8___boxed(lean_object* x_1) { +_start: +{ +uint8_t x_2; lean_object* x_3; +x_2 = l_instOfNatInt8(x_1); +lean_dec(x_1); +x_3 = lean_box(x_2); +return x_3; +} +} +static lean_object* _init_l_instNegInt8___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Int8_neg___boxed), 1, 0); +return x_1; +} +} +static lean_object* _init_l_instNegInt8() { +_start: +{ +lean_object* x_1; +x_1 = l_instNegInt8___closed__1; +return x_1; +} +} +LEAN_EXPORT lean_object* l_Int8_add___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 = lean_int8_add(x_3, x_4); +x_6 = lean_box(x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Int8_sub___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 = lean_int8_sub(x_3, x_4); +x_6 = lean_box(x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Int8_mul___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 = lean_int8_mul(x_3, x_4); +x_6 = lean_box(x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Int8_div___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 = lean_int8_div(x_3, x_4); +x_6 = lean_box(x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Int8_mod___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 = lean_int8_mod(x_3, x_4); +x_6 = lean_box(x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Int8_land___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 = lean_int8_land(x_3, x_4); +x_6 = lean_box(x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Int8_lor___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 = lean_int8_lor(x_3, x_4); +x_6 = lean_box(x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Int8_xor___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 = lean_int8_xor(x_3, x_4); +x_6 = lean_box(x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Int8_shiftLeft___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 = lean_int8_shift_left(x_3, x_4); +x_6 = lean_box(x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Int8_shiftRight___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 = lean_int8_shift_right(x_3, x_4); +x_6 = lean_box(x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Int8_complement___boxed(lean_object* x_1) { +_start: +{ +uint8_t x_2; uint8_t x_3; lean_object* x_4; +x_2 = lean_unbox(x_1); +lean_dec(x_1); +x_3 = lean_int8_complement(x_2); +x_4 = lean_box(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Int8_decEq___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 = lean_int8_dec_eq(x_3, x_4); +x_6 = lean_box(x_5); +return x_6; +} +} +static uint8_t _init_l_instInhabitedInt8___closed__1() { +_start: +{ +lean_object* x_1; uint8_t x_2; +x_1 = lean_unsigned_to_nat(0u); +x_2 = lean_int8_of_int(x_1); +return x_2; +} +} +static uint8_t _init_l_instInhabitedInt8() { +_start: +{ +uint8_t x_1; +x_1 = l_instInhabitedInt8___closed__1; +return x_1; +} +} +static lean_object* _init_l_instAddInt8___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Int8_add___boxed), 2, 0); +return x_1; +} +} +static lean_object* _init_l_instAddInt8() { +_start: +{ +lean_object* x_1; +x_1 = l_instAddInt8___closed__1; +return x_1; +} +} +static lean_object* _init_l_instSubInt8___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Int8_sub___boxed), 2, 0); +return x_1; +} +} +static lean_object* _init_l_instSubInt8() { +_start: +{ +lean_object* x_1; +x_1 = l_instSubInt8___closed__1; +return x_1; +} +} +static lean_object* _init_l_instMulInt8___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Int8_mul___boxed), 2, 0); +return x_1; +} +} +static lean_object* _init_l_instMulInt8() { +_start: +{ +lean_object* x_1; +x_1 = l_instMulInt8___closed__1; +return x_1; +} +} +static lean_object* _init_l_instModInt8___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Int8_mod___boxed), 2, 0); +return x_1; +} +} +static lean_object* _init_l_instModInt8() { +_start: +{ +lean_object* x_1; +x_1 = l_instModInt8___closed__1; +return x_1; +} +} +static lean_object* _init_l_instDivInt8___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Int8_div___boxed), 2, 0); +return x_1; +} +} +static lean_object* _init_l_instDivInt8() { +_start: +{ +lean_object* x_1; +x_1 = l_instDivInt8___closed__1; +return x_1; +} +} +static lean_object* _init_l_instLTInt8() { +_start: +{ +lean_object* x_1; +x_1 = lean_box(0); +return x_1; +} +} +static lean_object* _init_l_instLEInt8() { +_start: +{ +lean_object* x_1; +x_1 = lean_box(0); +return x_1; +} +} +static lean_object* _init_l_instComplementInt8___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Int8_complement___boxed), 1, 0); +return x_1; +} +} +static lean_object* _init_l_instComplementInt8() { +_start: +{ +lean_object* x_1; +x_1 = l_instComplementInt8___closed__1; +return x_1; +} +} +static lean_object* _init_l_instAndOpInt8___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Int8_land___boxed), 2, 0); +return x_1; +} +} +static lean_object* _init_l_instAndOpInt8() { +_start: +{ +lean_object* x_1; +x_1 = l_instAndOpInt8___closed__1; +return x_1; +} +} +static lean_object* _init_l_instOrOpInt8___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Int8_lor___boxed), 2, 0); +return x_1; +} +} +static lean_object* _init_l_instOrOpInt8() { +_start: +{ +lean_object* x_1; +x_1 = l_instOrOpInt8___closed__1; +return x_1; +} +} +static lean_object* _init_l_instXorInt8___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Int8_xor___boxed), 2, 0); +return x_1; +} +} +static lean_object* _init_l_instXorInt8() { +_start: +{ +lean_object* x_1; +x_1 = l_instXorInt8___closed__1; +return x_1; +} +} +static lean_object* _init_l_instShiftLeftInt8___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Int8_shiftLeft___boxed), 2, 0); +return x_1; +} +} +static lean_object* _init_l_instShiftLeftInt8() { +_start: +{ +lean_object* x_1; +x_1 = l_instShiftLeftInt8___closed__1; +return x_1; +} +} +static lean_object* _init_l_instShiftRightInt8___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Int8_shiftRight___boxed), 2, 0); +return x_1; +} +} +static lean_object* _init_l_instShiftRightInt8() { +_start: +{ +lean_object* x_1; +x_1 = l_instShiftRightInt8___closed__1; +return x_1; +} +} +LEAN_EXPORT uint8_t l_instDecidableEqInt8(uint8_t x_1, uint8_t x_2) { +_start: +{ +uint8_t x_3; +x_3 = lean_int8_dec_eq(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_instDecidableEqInt8___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_instDecidableEqInt8(x_3, x_4); +x_6 = lean_box(x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Int8_decLt___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 = lean_int8_dec_lt(x_3, x_4); +x_6 = lean_box(x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Int8_decLe___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 = lean_int8_dec_le(x_3, x_4); +x_6 = lean_box(x_5); +return x_6; +} +} +LEAN_EXPORT uint8_t l_instDecidableLtInt8(uint8_t x_1, uint8_t x_2) { +_start: +{ +uint8_t x_3; +x_3 = lean_int8_dec_lt(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_instDecidableLtInt8___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_instDecidableLtInt8(x_3, x_4); +x_6 = lean_box(x_5); +return x_6; +} +} +LEAN_EXPORT uint8_t l_instDecidableLeInt8(uint8_t x_1, uint8_t x_2) { +_start: +{ +uint8_t x_3; +x_3 = lean_int8_dec_le(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_instDecidableLeInt8___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_instDecidableLeInt8(x_3, x_4); +x_6 = lean_box(x_5); +return x_6; +} +} +LEAN_EXPORT uint8_t l_instMaxInt8(uint8_t x_1, uint8_t x_2) { +_start: +{ +uint8_t x_3; +x_3 = lean_int8_dec_le(x_1, x_2); +if (x_3 == 0) +{ +return x_1; +} +else +{ +return x_2; +} +} +} +LEAN_EXPORT lean_object* l_instMaxInt8___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_instMaxInt8(x_3, x_4); +x_6 = lean_box(x_5); +return x_6; +} +} +LEAN_EXPORT uint8_t l_instMinInt8(uint8_t x_1, uint8_t x_2) { +_start: +{ +uint8_t x_3; +x_3 = lean_int8_dec_le(x_1, x_2); +if (x_3 == 0) +{ +return x_2; +} +else +{ +return x_1; +} +} +} +LEAN_EXPORT lean_object* l_instMinInt8___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_instMinInt8(x_3, x_4); +x_6 = lean_box(x_5); +return x_6; +} +} +lean_object* initialize_Init_Data_UInt_Basic(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Init_Data_SInt_Basic(uint8_t builtin, lean_object* w) { +lean_object * res; +if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); +_G_initialized = true; +res = initialize_Init_Data_UInt_Basic(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +l_Int8_size = _init_l_Int8_size(); +lean_mark_persistent(l_Int8_size); +l_instToStringInt8___closed__1 = _init_l_instToStringInt8___closed__1(); +lean_mark_persistent(l_instToStringInt8___closed__1); +l_instToStringInt8___closed__2 = _init_l_instToStringInt8___closed__2(); +lean_mark_persistent(l_instToStringInt8___closed__2); +l_instNegInt8___closed__1 = _init_l_instNegInt8___closed__1(); +lean_mark_persistent(l_instNegInt8___closed__1); +l_instNegInt8 = _init_l_instNegInt8(); +lean_mark_persistent(l_instNegInt8); +l_instInhabitedInt8___closed__1 = _init_l_instInhabitedInt8___closed__1(); +l_instInhabitedInt8 = _init_l_instInhabitedInt8(); +l_instAddInt8___closed__1 = _init_l_instAddInt8___closed__1(); +lean_mark_persistent(l_instAddInt8___closed__1); +l_instAddInt8 = _init_l_instAddInt8(); +lean_mark_persistent(l_instAddInt8); +l_instSubInt8___closed__1 = _init_l_instSubInt8___closed__1(); +lean_mark_persistent(l_instSubInt8___closed__1); +l_instSubInt8 = _init_l_instSubInt8(); +lean_mark_persistent(l_instSubInt8); +l_instMulInt8___closed__1 = _init_l_instMulInt8___closed__1(); +lean_mark_persistent(l_instMulInt8___closed__1); +l_instMulInt8 = _init_l_instMulInt8(); +lean_mark_persistent(l_instMulInt8); +l_instModInt8___closed__1 = _init_l_instModInt8___closed__1(); +lean_mark_persistent(l_instModInt8___closed__1); +l_instModInt8 = _init_l_instModInt8(); +lean_mark_persistent(l_instModInt8); +l_instDivInt8___closed__1 = _init_l_instDivInt8___closed__1(); +lean_mark_persistent(l_instDivInt8___closed__1); +l_instDivInt8 = _init_l_instDivInt8(); +lean_mark_persistent(l_instDivInt8); +l_instLTInt8 = _init_l_instLTInt8(); +lean_mark_persistent(l_instLTInt8); +l_instLEInt8 = _init_l_instLEInt8(); +lean_mark_persistent(l_instLEInt8); +l_instComplementInt8___closed__1 = _init_l_instComplementInt8___closed__1(); +lean_mark_persistent(l_instComplementInt8___closed__1); +l_instComplementInt8 = _init_l_instComplementInt8(); +lean_mark_persistent(l_instComplementInt8); +l_instAndOpInt8___closed__1 = _init_l_instAndOpInt8___closed__1(); +lean_mark_persistent(l_instAndOpInt8___closed__1); +l_instAndOpInt8 = _init_l_instAndOpInt8(); +lean_mark_persistent(l_instAndOpInt8); +l_instOrOpInt8___closed__1 = _init_l_instOrOpInt8___closed__1(); +lean_mark_persistent(l_instOrOpInt8___closed__1); +l_instOrOpInt8 = _init_l_instOrOpInt8(); +lean_mark_persistent(l_instOrOpInt8); +l_instXorInt8___closed__1 = _init_l_instXorInt8___closed__1(); +lean_mark_persistent(l_instXorInt8___closed__1); +l_instXorInt8 = _init_l_instXorInt8(); +lean_mark_persistent(l_instXorInt8); +l_instShiftLeftInt8___closed__1 = _init_l_instShiftLeftInt8___closed__1(); +lean_mark_persistent(l_instShiftLeftInt8___closed__1); +l_instShiftLeftInt8 = _init_l_instShiftLeftInt8(); +lean_mark_persistent(l_instShiftLeftInt8); +l_instShiftRightInt8___closed__1 = _init_l_instShiftRightInt8___closed__1(); +lean_mark_persistent(l_instShiftRightInt8___closed__1); +l_instShiftRightInt8 = _init_l_instShiftRightInt8(); +lean_mark_persistent(l_instShiftRightInt8); +return lean_io_result_mk_ok(lean_box(0)); +} +#ifdef __cplusplus +} +#endif diff --git a/stage0/stdlib/Init/Data/String/Basic.c b/stage0/stdlib/Init/Data/String/Basic.c index 6a968c286229..33da3bd3c40e 100644 --- a/stage0/stdlib/Init/Data/String/Basic.c +++ b/stage0/stdlib/Init/Data/String/Basic.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Init.Data.String.Basic -// Imports: Init.Data.List.Basic Init.Data.Char.Basic Init.Data.Option.Basic +// Imports: Init.Data.List.Basic Init.Data.Char.Basic #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -6878,29 +6878,39 @@ return x_6; LEAN_EXPORT lean_object* l_String_dropPrefix_x3f(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; x_3 = lean_string_utf8_byte_size(x_1); x_4 = lean_unsigned_to_nat(0u); x_5 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_5, 0, x_1); lean_ctor_set(x_5, 1, x_4); lean_ctor_set(x_5, 2, x_3); -x_6 = l_Substring_dropPrefix_x3f(x_5, x_2); -return x_6; +x_6 = lean_string_utf8_byte_size(x_2); +x_7 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_7, 0, x_2); +lean_ctor_set(x_7, 1, x_4); +lean_ctor_set(x_7, 2, x_6); +x_8 = l_Substring_dropPrefix_x3f(x_5, x_7); +return x_8; } } LEAN_EXPORT lean_object* l_String_dropSuffix_x3f(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; x_3 = lean_string_utf8_byte_size(x_1); x_4 = lean_unsigned_to_nat(0u); x_5 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_5, 0, x_1); lean_ctor_set(x_5, 1, x_4); lean_ctor_set(x_5, 2, x_3); -x_6 = l_Substring_dropSuffix_x3f(x_5, x_2); -return x_6; +x_6 = lean_string_utf8_byte_size(x_2); +x_7 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_7, 0, x_2); +lean_ctor_set(x_7, 1, x_4); +lean_ctor_set(x_7, 2, x_6); +x_8 = l_Substring_dropSuffix_x3f(x_5, x_7); +return x_8; } } LEAN_EXPORT lean_object* l_String_stripPrefix(lean_object* x_1, lean_object* x_2) { @@ -7116,7 +7126,6 @@ return x_6; } lean_object* initialize_Init_Data_List_Basic(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_Char_Basic(uint8_t builtin, lean_object*); -lean_object* initialize_Init_Data_Option_Basic(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Init_Data_String_Basic(uint8_t builtin, lean_object* w) { lean_object * res; @@ -7128,9 +7137,6 @@ lean_dec_ref(res); res = initialize_Init_Data_Char_Basic(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -res = initialize_Init_Data_Option_Basic(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); l_String_instOfNatPos = _init_l_String_instOfNatPos(); lean_mark_persistent(l_String_instOfNatPos); l_String_instLT = _init_l_String_instLT(); diff --git a/stage0/stdlib/Init/Data/Sum.c b/stage0/stdlib/Init/Data/Sum.c index a7f39344c8b0..b8a0e444fc3a 100644 --- a/stage0/stdlib/Init/Data/Sum.c +++ b/stage0/stdlib/Init/Data/Sum.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Init.Data.Sum -// Imports: Init.Core +// Imports: Init.Data.Sum.Basic Init.Data.Sum.Lemmas #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -13,268 +13,17 @@ #ifdef __cplusplus extern "C" { #endif -LEAN_EXPORT lean_object* l_Sum_getRight_x3f(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Data_Sum_0__Sum_decEqSum____x40_Init_Data_Sum___hyg_4____rarg(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Sum_getLeft_x3f(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Sum_getRight_x3f___rarg(lean_object*); -LEAN_EXPORT lean_object* l_Sum_instDecidableEq(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Data_Sum_0__Sum_decEqSum____x40_Init_Data_Sum___hyg_4_(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Sum_getLeft_x3f___rarg(lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Data_Sum_0__Sum_beqSum____x40_Init_Data_Sum___hyg_242_(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Data_Sum_0__Sum_beqSum____x40_Init_Data_Sum___hyg_242____rarg(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Sum_instBEq(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Sum_instBEq___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Sum_instDecidableEq___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Data_Sum_0__Sum_decEqSum____x40_Init_Data_Sum___hyg_4____rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -if (lean_obj_tag(x_3) == 0) -{ -lean_dec(x_2); -if (lean_obj_tag(x_4) == 0) -{ -lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_5 = lean_ctor_get(x_3, 0); -lean_inc(x_5); -lean_dec(x_3); -x_6 = lean_ctor_get(x_4, 0); -lean_inc(x_6); -lean_dec(x_4); -x_7 = lean_apply_2(x_1, x_5, x_6); -return x_7; -} -else -{ -uint8_t x_8; lean_object* x_9; -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_8 = 0; -x_9 = lean_box(x_8); -return x_9; -} -} -else -{ -lean_dec(x_1); -if (lean_obj_tag(x_4) == 0) -{ -uint8_t x_10; lean_object* x_11; -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_10 = 0; -x_11 = lean_box(x_10); -return x_11; -} -else -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_12 = lean_ctor_get(x_3, 0); -lean_inc(x_12); -lean_dec(x_3); -x_13 = lean_ctor_get(x_4, 0); -lean_inc(x_13); -lean_dec(x_4); -x_14 = lean_apply_2(x_2, x_12, x_13); -return x_14; -} -} -} -} -LEAN_EXPORT lean_object* l___private_Init_Data_Sum_0__Sum_decEqSum____x40_Init_Data_Sum___hyg_4_(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l___private_Init_Data_Sum_0__Sum_decEqSum____x40_Init_Data_Sum___hyg_4____rarg), 4, 0); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Sum_instDecidableEq___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -lean_object* x_5; -x_5 = l___private_Init_Data_Sum_0__Sum_decEqSum____x40_Init_Data_Sum___hyg_4____rarg(x_1, x_2, x_3, x_4); -return x_5; -} -} -LEAN_EXPORT lean_object* l_Sum_instDecidableEq(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Sum_instDecidableEq___rarg), 4, 0); -return x_3; -} -} -LEAN_EXPORT lean_object* l___private_Init_Data_Sum_0__Sum_beqSum____x40_Init_Data_Sum___hyg_242____rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -if (lean_obj_tag(x_3) == 0) -{ -lean_dec(x_2); -if (lean_obj_tag(x_4) == 0) -{ -lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_5 = lean_ctor_get(x_3, 0); -lean_inc(x_5); -lean_dec(x_3); -x_6 = lean_ctor_get(x_4, 0); -lean_inc(x_6); -lean_dec(x_4); -x_7 = lean_apply_2(x_1, x_5, x_6); -return x_7; -} -else -{ -uint8_t x_8; lean_object* x_9; -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_8 = 0; -x_9 = lean_box(x_8); -return x_9; -} -} -else -{ -lean_dec(x_1); -if (lean_obj_tag(x_4) == 0) -{ -uint8_t x_10; lean_object* x_11; -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_10 = 0; -x_11 = lean_box(x_10); -return x_11; -} -else -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_12 = lean_ctor_get(x_3, 0); -lean_inc(x_12); -lean_dec(x_3); -x_13 = lean_ctor_get(x_4, 0); -lean_inc(x_13); -lean_dec(x_4); -x_14 = lean_apply_2(x_2, x_12, x_13); -return x_14; -} -} -} -} -LEAN_EXPORT lean_object* l___private_Init_Data_Sum_0__Sum_beqSum____x40_Init_Data_Sum___hyg_242_(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l___private_Init_Data_Sum_0__Sum_beqSum____x40_Init_Data_Sum___hyg_242____rarg), 4, 0); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Sum_instBEq___rarg(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l___private_Init_Data_Sum_0__Sum_beqSum____x40_Init_Data_Sum___hyg_242____rarg), 4, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Sum_instBEq(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Sum_instBEq___rarg), 2, 0); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Sum_getLeft_x3f___rarg(lean_object* x_1) { -_start: -{ -if (lean_obj_tag(x_1) == 0) -{ -uint8_t x_2; -x_2 = !lean_is_exclusive(x_1); -if (x_2 == 0) -{ -lean_ctor_set_tag(x_1, 1); -return x_1; -} -else -{ -lean_object* x_3; lean_object* x_4; -x_3 = lean_ctor_get(x_1, 0); -lean_inc(x_3); -lean_dec(x_1); -x_4 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_4, 0, x_3); -return x_4; -} -} -else -{ -lean_object* x_5; -lean_dec(x_1); -x_5 = lean_box(0); -return x_5; -} -} -} -LEAN_EXPORT lean_object* l_Sum_getLeft_x3f(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Sum_getLeft_x3f___rarg), 1, 0); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Sum_getRight_x3f___rarg(lean_object* x_1) { -_start: -{ -if (lean_obj_tag(x_1) == 0) -{ -lean_object* x_2; -lean_dec(x_1); -x_2 = lean_box(0); -return x_2; -} -else -{ -uint8_t x_3; -x_3 = !lean_is_exclusive(x_1); -if (x_3 == 0) -{ -return x_1; -} -else -{ -lean_object* x_4; lean_object* x_5; -x_4 = lean_ctor_get(x_1, 0); -lean_inc(x_4); -lean_dec(x_1); -x_5 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_5, 0, x_4); -return x_5; -} -} -} -} -LEAN_EXPORT lean_object* l_Sum_getRight_x3f(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Sum_getRight_x3f___rarg), 1, 0); -return x_3; -} -} -lean_object* initialize_Init_Core(uint8_t builtin, lean_object*); +lean_object* initialize_Init_Data_Sum_Basic(uint8_t builtin, lean_object*); +lean_object* initialize_Init_Data_Sum_Lemmas(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Init_Data_Sum(uint8_t builtin, lean_object* w) { lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init_Core(builtin, lean_io_mk_world()); +res = initialize_Init_Data_Sum_Basic(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Init_Data_Sum_Lemmas(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); return lean_io_result_mk_ok(lean_box(0)); diff --git a/stage0/stdlib/Init/Data/Sum/Basic.c b/stage0/stdlib/Init/Data/Sum/Basic.c new file mode 100644 index 000000000000..60e8434ccdb1 --- /dev/null +++ b/stage0/stdlib/Init/Data/Sum/Basic.c @@ -0,0 +1,676 @@ +// Lean compiler output +// Module: Init.Data.Sum.Basic +// Imports: Init.PropLemmas +#include +#if defined(__clang__) +#pragma clang diagnostic ignored "-Wunused-parameter" +#pragma clang diagnostic ignored "-Wunused-label" +#elif defined(__GNUC__) && !defined(__CLANG__) +#pragma GCC diagnostic ignored "-Wunused-parameter" +#pragma GCC diagnostic ignored "-Wunused-label" +#pragma GCC diagnostic ignored "-Wunused-but-set-variable" +#endif +#ifdef __cplusplus +extern "C" { +#endif +LEAN_EXPORT lean_object* l___private_Init_Data_Sum_Basic_0__Sum_decEqSum____x40_Init_Data_Sum_Basic___hyg_5_(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_isRight(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_swap(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_getRight_x3f(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_map___rarg___lambda__1(lean_object*); +LEAN_EXPORT lean_object* l_Sum_map(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_getRight___rarg___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_getLeft(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_getLeft_x3f(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_map___rarg___lambda__2(lean_object*); +LEAN_EXPORT lean_object* l_Sum_getRight_x3f___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Sum_instDecidableLiftRel(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_instDecidableEq(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_isLeft___rarg___boxed(lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Sum_Basic_0__Sum_beqSum____x40_Init_Data_Sum_Basic___hyg_243_(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_getRight(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_map___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_swap___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Sum_elim___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_getLeft_x3f___rarg(lean_object*); +static lean_object* l_Sum_map___rarg___closed__1; +LEAN_EXPORT uint8_t l_Sum_isLeft___rarg(lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Sum_Basic_0__Sum_decEqSum____x40_Init_Data_Sum_Basic___hyg_5____rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_instDecidableLiftRel___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_isRight___rarg___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Sum_getLeft___rarg___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_instDecidableRelSumLex___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Sum_Basic_0__Sum_beqSum____x40_Init_Data_Sum_Basic___hyg_243____rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_instDecidableRelSumLex(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_isLeft(lean_object*, lean_object*); +lean_object* l_Function_comp___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_instBEq(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_instBEq___rarg(lean_object*, lean_object*); +static lean_object* l_Sum_map___rarg___closed__2; +LEAN_EXPORT uint8_t l_Sum_isRight___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Sum_instDecidableEq___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_getRight___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_elim(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_getLeft___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Sum_Basic_0__Sum_decEqSum____x40_Init_Data_Sum_Basic___hyg_5____rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +if (lean_obj_tag(x_3) == 0) +{ +lean_dec(x_2); +if (lean_obj_tag(x_4) == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_5 = lean_ctor_get(x_3, 0); +lean_inc(x_5); +lean_dec(x_3); +x_6 = lean_ctor_get(x_4, 0); +lean_inc(x_6); +lean_dec(x_4); +x_7 = lean_apply_2(x_1, x_5, x_6); +return x_7; +} +else +{ +uint8_t x_8; lean_object* x_9; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_8 = 0; +x_9 = lean_box(x_8); +return x_9; +} +} +else +{ +lean_dec(x_1); +if (lean_obj_tag(x_4) == 0) +{ +uint8_t x_10; lean_object* x_11; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_10 = 0; +x_11 = lean_box(x_10); +return x_11; +} +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_3, 0); +lean_inc(x_12); +lean_dec(x_3); +x_13 = lean_ctor_get(x_4, 0); +lean_inc(x_13); +lean_dec(x_4); +x_14 = lean_apply_2(x_2, x_12, x_13); +return x_14; +} +} +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Sum_Basic_0__Sum_decEqSum____x40_Init_Data_Sum_Basic___hyg_5_(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l___private_Init_Data_Sum_Basic_0__Sum_decEqSum____x40_Init_Data_Sum_Basic___hyg_5____rarg), 4, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Sum_instDecidableEq___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l___private_Init_Data_Sum_Basic_0__Sum_decEqSum____x40_Init_Data_Sum_Basic___hyg_5____rarg(x_1, x_2, x_3, x_4); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Sum_instDecidableEq(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Sum_instDecidableEq___rarg), 4, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Sum_Basic_0__Sum_beqSum____x40_Init_Data_Sum_Basic___hyg_243____rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +if (lean_obj_tag(x_3) == 0) +{ +lean_dec(x_2); +if (lean_obj_tag(x_4) == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_5 = lean_ctor_get(x_3, 0); +lean_inc(x_5); +lean_dec(x_3); +x_6 = lean_ctor_get(x_4, 0); +lean_inc(x_6); +lean_dec(x_4); +x_7 = lean_apply_2(x_1, x_5, x_6); +return x_7; +} +else +{ +uint8_t x_8; lean_object* x_9; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_8 = 0; +x_9 = lean_box(x_8); +return x_9; +} +} +else +{ +lean_dec(x_1); +if (lean_obj_tag(x_4) == 0) +{ +uint8_t x_10; lean_object* x_11; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_10 = 0; +x_11 = lean_box(x_10); +return x_11; +} +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_3, 0); +lean_inc(x_12); +lean_dec(x_3); +x_13 = lean_ctor_get(x_4, 0); +lean_inc(x_13); +lean_dec(x_4); +x_14 = lean_apply_2(x_2, x_12, x_13); +return x_14; +} +} +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Sum_Basic_0__Sum_beqSum____x40_Init_Data_Sum_Basic___hyg_243_(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l___private_Init_Data_Sum_Basic_0__Sum_beqSum____x40_Init_Data_Sum_Basic___hyg_243____rarg), 4, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Sum_instBEq___rarg(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l___private_Init_Data_Sum_Basic_0__Sum_beqSum____x40_Init_Data_Sum_Basic___hyg_243____rarg), 4, 2); +lean_closure_set(x_3, 0, x_1); +lean_closure_set(x_3, 1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Sum_instBEq(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Sum_instBEq___rarg), 2, 0); +return x_3; +} +} +LEAN_EXPORT uint8_t l_Sum_isLeft___rarg(lean_object* x_1) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +uint8_t x_2; +x_2 = 1; +return x_2; +} +else +{ +uint8_t x_3; +x_3 = 0; +return x_3; +} +} +} +LEAN_EXPORT lean_object* l_Sum_isLeft(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Sum_isLeft___rarg___boxed), 1, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Sum_isLeft___rarg___boxed(lean_object* x_1) { +_start: +{ +uint8_t x_2; lean_object* x_3; +x_2 = l_Sum_isLeft___rarg(x_1); +lean_dec(x_1); +x_3 = lean_box(x_2); +return x_3; +} +} +LEAN_EXPORT uint8_t l_Sum_isRight___rarg(lean_object* x_1) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +uint8_t x_2; +x_2 = 0; +return x_2; +} +else +{ +uint8_t x_3; +x_3 = 1; +return x_3; +} +} +} +LEAN_EXPORT lean_object* l_Sum_isRight(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Sum_isRight___rarg___boxed), 1, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Sum_isRight___rarg___boxed(lean_object* x_1) { +_start: +{ +uint8_t x_2; lean_object* x_3; +x_2 = l_Sum_isRight___rarg(x_1); +lean_dec(x_1); +x_3 = lean_box(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Sum_getLeft___rarg(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_ctor_get(x_1, 0); +lean_inc(x_3); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Sum_getLeft(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Sum_getLeft___rarg___boxed), 2, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Sum_getLeft___rarg___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Sum_getLeft___rarg(x_1, x_2); +lean_dec(x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Sum_getRight___rarg(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_ctor_get(x_1, 0); +lean_inc(x_3); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Sum_getRight(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Sum_getRight___rarg___boxed), 2, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Sum_getRight___rarg___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Sum_getRight___rarg(x_1, x_2); +lean_dec(x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Sum_getLeft_x3f___rarg(lean_object* x_1) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +uint8_t x_2; +x_2 = !lean_is_exclusive(x_1); +if (x_2 == 0) +{ +lean_ctor_set_tag(x_1, 1); +return x_1; +} +else +{ +lean_object* x_3; lean_object* x_4; +x_3 = lean_ctor_get(x_1, 0); +lean_inc(x_3); +lean_dec(x_1); +x_4 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_4, 0, x_3); +return x_4; +} +} +else +{ +lean_object* x_5; +lean_dec(x_1); +x_5 = lean_box(0); +return x_5; +} +} +} +LEAN_EXPORT lean_object* l_Sum_getLeft_x3f(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Sum_getLeft_x3f___rarg), 1, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Sum_getRight_x3f___rarg(lean_object* x_1) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_2; +lean_dec(x_1); +x_2 = lean_box(0); +return x_2; +} +else +{ +uint8_t x_3; +x_3 = !lean_is_exclusive(x_1); +if (x_3 == 0) +{ +return x_1; +} +else +{ +lean_object* x_4; lean_object* x_5; +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_5, 0, x_4); +return x_5; +} +} +} +} +LEAN_EXPORT lean_object* l_Sum_getRight_x3f(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Sum_getRight_x3f___rarg), 1, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Sum_elim___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +if (lean_obj_tag(x_3) == 0) +{ +lean_object* x_4; lean_object* x_5; +lean_dec(x_2); +x_4 = lean_ctor_get(x_3, 0); +lean_inc(x_4); +lean_dec(x_3); +x_5 = lean_apply_1(x_1, x_4); +return x_5; +} +else +{ +lean_object* x_6; lean_object* x_7; +lean_dec(x_1); +x_6 = lean_ctor_get(x_3, 0); +lean_inc(x_6); +lean_dec(x_3); +x_7 = lean_apply_1(x_2, x_6); +return x_7; +} +} +} +LEAN_EXPORT lean_object* l_Sum_elim(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = lean_alloc_closure((void*)(l_Sum_elim___rarg), 3, 0); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Sum_map___rarg___lambda__1(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Sum_map___rarg___lambda__2(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Sum_map___rarg___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Sum_map___rarg___lambda__1), 1, 0); +return x_1; +} +} +static lean_object* _init_l_Sum_map___rarg___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Sum_map___rarg___lambda__2), 1, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Sum_map___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_4 = l_Sum_map___rarg___closed__1; +x_5 = lean_alloc_closure((void*)(l_Function_comp___rarg), 3, 2); +lean_closure_set(x_5, 0, x_4); +lean_closure_set(x_5, 1, x_1); +x_6 = l_Sum_map___rarg___closed__2; +x_7 = lean_alloc_closure((void*)(l_Function_comp___rarg), 3, 2); +lean_closure_set(x_7, 0, x_6); +lean_closure_set(x_7, 1, x_2); +x_8 = l_Sum_elim___rarg(x_5, x_7, x_3); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Sum_map(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = lean_alloc_closure((void*)(l_Sum_map___rarg), 3, 0); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Sum_swap___rarg(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_2 = l_Sum_map___rarg___closed__2; +x_3 = l_Sum_map___rarg___closed__1; +x_4 = l_Sum_elim___rarg(x_2, x_3, x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Sum_swap(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Sum_swap___rarg), 1, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Sum_instDecidableLiftRel___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +if (lean_obj_tag(x_3) == 0) +{ +lean_dec(x_2); +if (lean_obj_tag(x_4) == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_5 = lean_ctor_get(x_3, 0); +lean_inc(x_5); +lean_dec(x_3); +x_6 = lean_ctor_get(x_4, 0); +lean_inc(x_6); +lean_dec(x_4); +x_7 = lean_apply_2(x_1, x_5, x_6); +return x_7; +} +else +{ +uint8_t x_8; lean_object* x_9; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_8 = 0; +x_9 = lean_box(x_8); +return x_9; +} +} +else +{ +lean_dec(x_1); +if (lean_obj_tag(x_4) == 0) +{ +uint8_t x_10; lean_object* x_11; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_10 = 0; +x_11 = lean_box(x_10); +return x_11; +} +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_3, 0); +lean_inc(x_12); +lean_dec(x_3); +x_13 = lean_ctor_get(x_4, 0); +lean_inc(x_13); +lean_dec(x_4); +x_14 = lean_apply_2(x_2, x_12, x_13); +return x_14; +} +} +} +} +LEAN_EXPORT lean_object* l_Sum_instDecidableLiftRel(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; +x_7 = lean_alloc_closure((void*)(l_Sum_instDecidableLiftRel___rarg), 4, 0); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Sum_instDecidableRelSumLex___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +if (lean_obj_tag(x_3) == 0) +{ +lean_dec(x_2); +if (lean_obj_tag(x_4) == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_5 = lean_ctor_get(x_3, 0); +lean_inc(x_5); +lean_dec(x_3); +x_6 = lean_ctor_get(x_4, 0); +lean_inc(x_6); +lean_dec(x_4); +x_7 = lean_apply_2(x_1, x_5, x_6); +return x_7; +} +else +{ +uint8_t x_8; lean_object* x_9; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_8 = 1; +x_9 = lean_box(x_8); +return x_9; +} +} +else +{ +lean_dec(x_1); +if (lean_obj_tag(x_4) == 0) +{ +uint8_t x_10; lean_object* x_11; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_10 = 0; +x_11 = lean_box(x_10); +return x_11; +} +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_3, 0); +lean_inc(x_12); +lean_dec(x_3); +x_13 = lean_ctor_get(x_4, 0); +lean_inc(x_13); +lean_dec(x_4); +x_14 = lean_apply_2(x_2, x_12, x_13); +return x_14; +} +} +} +} +LEAN_EXPORT lean_object* l_Sum_instDecidableRelSumLex(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = lean_alloc_closure((void*)(l_Sum_instDecidableRelSumLex___rarg), 4, 0); +return x_5; +} +} +lean_object* initialize_Init_PropLemmas(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Init_Data_Sum_Basic(uint8_t builtin, lean_object* w) { +lean_object * res; +if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); +_G_initialized = true; +res = initialize_Init_PropLemmas(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +l_Sum_map___rarg___closed__1 = _init_l_Sum_map___rarg___closed__1(); +lean_mark_persistent(l_Sum_map___rarg___closed__1); +l_Sum_map___rarg___closed__2 = _init_l_Sum_map___rarg___closed__2(); +lean_mark_persistent(l_Sum_map___rarg___closed__2); +return lean_io_result_mk_ok(lean_box(0)); +} +#ifdef __cplusplus +} +#endif diff --git a/stage0/stdlib/Init/Data/Sum/Lemmas.c b/stage0/stdlib/Init/Data/Sum/Lemmas.c new file mode 100644 index 000000000000..5bd791f44fd4 --- /dev/null +++ b/stage0/stdlib/Init/Data/Sum/Lemmas.c @@ -0,0 +1,103 @@ +// Lean compiler output +// Module: Init.Data.Sum.Lemmas +// Imports: Init.Data.Sum.Basic Init.Ext +#include +#if defined(__clang__) +#pragma clang diagnostic ignored "-Wunused-parameter" +#pragma clang diagnostic ignored "-Wunused-label" +#elif defined(__GNUC__) && !defined(__CLANG__) +#pragma GCC diagnostic ignored "-Wunused-parameter" +#pragma GCC diagnostic ignored "-Wunused-label" +#pragma GCC diagnostic ignored "-Wunused-but-set-variable" +#endif +#ifdef __cplusplus +extern "C" { +#endif +LEAN_EXPORT lean_object* l___private_Init_Data_Sum_Lemmas_0__Sum_getRight_x3f_match__1_splitter(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Sum_Lemmas_0__Sum_isLeft_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Sum_Lemmas_0__Sum_getRight_x3f_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Sum_Lemmas_0__Sum_isLeft_match__1_splitter(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Sum_Lemmas_0__Sum_isLeft_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_4; lean_object* x_5; +lean_dec(x_3); +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_apply_1(x_2, x_4); +return x_5; +} +else +{ +lean_object* x_6; lean_object* x_7; +lean_dec(x_2); +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +lean_dec(x_1); +x_7 = lean_apply_1(x_3, x_6); +return x_7; +} +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Sum_Lemmas_0__Sum_isLeft_match__1_splitter(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = lean_alloc_closure((void*)(l___private_Init_Data_Sum_Lemmas_0__Sum_isLeft_match__1_splitter___rarg), 3, 0); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Sum_Lemmas_0__Sum_getRight_x3f_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_4; lean_object* x_5; +lean_dec(x_2); +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_apply_1(x_3, x_4); +return x_5; +} +else +{ +lean_object* x_6; lean_object* x_7; +lean_dec(x_3); +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +lean_dec(x_1); +x_7 = lean_apply_1(x_2, x_6); +return x_7; +} +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Sum_Lemmas_0__Sum_getRight_x3f_match__1_splitter(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = lean_alloc_closure((void*)(l___private_Init_Data_Sum_Lemmas_0__Sum_getRight_x3f_match__1_splitter___rarg), 3, 0); +return x_4; +} +} +lean_object* initialize_Init_Data_Sum_Basic(uint8_t builtin, lean_object*); +lean_object* initialize_Init_Ext(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Init_Data_Sum_Lemmas(uint8_t builtin, lean_object* w) { +lean_object * res; +if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); +_G_initialized = true; +res = initialize_Init_Data_Sum_Basic(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Init_Ext(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +return lean_io_result_mk_ok(lean_box(0)); +} +#ifdef __cplusplus +} +#endif diff --git a/stage0/stdlib/Init/Data/ToString/Basic.c b/stage0/stdlib/Init/Data/ToString/Basic.c index b8baf8777c29..8bf5db239636 100644 --- a/stage0/stdlib/Init/Data/ToString/Basic.c +++ b/stage0/stdlib/Init/Data/ToString/Basic.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Init.Data.ToString.Basic -// Imports: Init.Data.String.Basic Init.Data.UInt.BasicAux Init.Data.Nat.Div Init.Data.Repr Init.Data.Int.Basic Init.Data.Format.Basic Init.Control.Id Init.Control.Option +// Imports: Init.Data.Repr Init.Data.Option.Basic #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -1527,41 +1527,17 @@ lean_dec(x_4); return x_5; } } -lean_object* initialize_Init_Data_String_Basic(uint8_t builtin, lean_object*); -lean_object* initialize_Init_Data_UInt_BasicAux(uint8_t builtin, lean_object*); -lean_object* initialize_Init_Data_Nat_Div(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_Repr(uint8_t builtin, lean_object*); -lean_object* initialize_Init_Data_Int_Basic(uint8_t builtin, lean_object*); -lean_object* initialize_Init_Data_Format_Basic(uint8_t builtin, lean_object*); -lean_object* initialize_Init_Control_Id(uint8_t builtin, lean_object*); -lean_object* initialize_Init_Control_Option(uint8_t builtin, lean_object*); +lean_object* initialize_Init_Data_Option_Basic(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Init_Data_ToString_Basic(uint8_t builtin, lean_object* w) { lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init_Data_String_Basic(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -res = initialize_Init_Data_UInt_BasicAux(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -res = initialize_Init_Data_Nat_Div(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Init_Data_Repr(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -res = initialize_Init_Data_Int_Basic(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -res = initialize_Init_Data_Format_Basic(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -res = initialize_Init_Control_Id(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -res = initialize_Init_Control_Option(builtin, lean_io_mk_world()); +res = initialize_Init_Data_Option_Basic(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); l_instToStringBool___closed__1 = _init_l_instToStringBool___closed__1(); diff --git a/stage0/stdlib/Init/Data/UInt/Lemmas.c b/stage0/stdlib/Init/Data/UInt/Lemmas.c index 227d1f866b53..7f700bb493ec 100644 --- a/stage0/stdlib/Init/Data/UInt/Lemmas.c +++ b/stage0/stdlib/Init/Data/UInt/Lemmas.c @@ -82,6 +82,7 @@ static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDe static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__179; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__356; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__442; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__515; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__353; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__24; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__190; @@ -99,9 +100,11 @@ static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDe static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__504; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__189; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__192; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__524; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__134; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__46; static lean_object* l_commandDeclare__uint__theorems_____closed__9; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__518; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__202; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__368; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__309; @@ -227,7 +230,9 @@ static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDe static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__100; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__425; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__108; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__512; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__341; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__507; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__80; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__416; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__473; @@ -241,6 +246,7 @@ static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDe static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__62; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__54; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__453; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__522; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__175; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__278; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__333; @@ -252,6 +258,7 @@ static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDe static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__139; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__355; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__43; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__510; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__437; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__66; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__57; @@ -293,6 +300,7 @@ static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDe static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__237; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__424; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__17; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__511; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__338; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__29; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__115; @@ -300,10 +308,12 @@ static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDe static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__432; static lean_object* l_commandDeclare__uint__theorems_____closed__6; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__509; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__295; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__55; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__495; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__77; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__505; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__114; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__307; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__92; @@ -341,8 +351,10 @@ static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDe static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__489; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__409; LEAN_EXPORT lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1(lean_object*, lean_object*, lean_object*); +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__519; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__185; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__394; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__506; static lean_object* l_commandDeclare__uint__theorems_____closed__2; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__397; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__301; @@ -409,12 +421,14 @@ static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDe lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__75; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__222; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__516; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__122; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__212; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__73; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__328; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__176; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__369; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__513; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__188; lean_object* l_Lean_Syntax_node7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__344; @@ -444,6 +458,7 @@ static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDe static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__131; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__106; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__438; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__525; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__161; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__476; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__314; @@ -453,8 +468,10 @@ static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDe static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__229; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__197; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__474; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__521; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__383; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__388; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__520; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__444; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__121; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__457; @@ -488,7 +505,9 @@ static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDe static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__27; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__198; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__195; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__523; lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__514; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__402; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__396; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__289; @@ -508,9 +527,11 @@ static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDe static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__349; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__155; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__332; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__517; LEAN_EXPORT uint8_t l_UInt8_instInhabited; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__20; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__249; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__508; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__299; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__231; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__311; @@ -5251,18 +5272,208 @@ static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__com _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("end", 3, 3); +x_1 = lean_mk_string_unchecked("val_ofNat", 9, 9); return x_1; } } static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__504() { _start: { +lean_object* x_1; lean_object* x_2; +x_1 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__503; +x_2 = l_String_toSubstring_x27(x_1); +return x_2; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__505() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__503; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__506() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("noindex", 7, 7); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__507() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__3; +x_2 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__4; +x_3 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__15; +x_4 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__506; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__508() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("no_index", 8, 8); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__509() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("OfNat.ofNat", 11, 11); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__510() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__509; +x_2 = l_String_toSubstring_x27(x_1); +return x_2; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__511() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("OfNat", 5, 5); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__512() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__511; +x_2 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__168; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__513() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("toBitVec_ofNat", 14, 14); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__514() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__513; +x_2 = l_String_toSubstring_x27(x_1); +return x_2; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__515() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__513; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__516() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__90; +x_2 = l_String_toSubstring_x27(x_1); +return x_2; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__517() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__90; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__518() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("BitVec.ofNat", 12, 12); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__519() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__518; +x_2 = l_String_toSubstring_x27(x_1); +return x_2; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__520() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__249; +x_2 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__168; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__521() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mk_ofNat", 8, 8); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__522() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__521; +x_2 = l_String_toSubstring_x27(x_1); +return x_2; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__523() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__521; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__524() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("end", 3, 3); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__525() { +_start: +{ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__3; x_2 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__4; x_3 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__5; -x_4 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__503; +x_4 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__524; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } @@ -5286,7 +5497,7 @@ return x_7; } else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; lean_object* x_286; lean_object* x_287; lean_object* x_288; lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; lean_object* x_294; lean_object* x_295; lean_object* x_296; lean_object* x_297; lean_object* x_298; lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; lean_object* x_307; lean_object* x_308; lean_object* x_309; lean_object* x_310; lean_object* x_311; lean_object* x_312; lean_object* x_313; lean_object* x_314; lean_object* x_315; lean_object* x_316; lean_object* x_317; lean_object* x_318; lean_object* x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; lean_object* x_324; lean_object* x_325; lean_object* x_326; lean_object* x_327; lean_object* x_328; lean_object* x_329; lean_object* x_330; lean_object* x_331; lean_object* x_332; lean_object* x_333; lean_object* x_334; lean_object* x_335; lean_object* x_336; lean_object* x_337; lean_object* x_338; lean_object* x_339; lean_object* x_340; lean_object* x_341; lean_object* x_342; lean_object* x_343; lean_object* x_344; lean_object* x_345; lean_object* x_346; lean_object* x_347; lean_object* x_348; lean_object* x_349; lean_object* x_350; lean_object* x_351; lean_object* x_352; lean_object* x_353; lean_object* x_354; lean_object* x_355; lean_object* x_356; lean_object* x_357; lean_object* x_358; lean_object* x_359; lean_object* x_360; lean_object* x_361; lean_object* x_362; lean_object* x_363; lean_object* x_364; lean_object* x_365; lean_object* x_366; lean_object* x_367; lean_object* x_368; lean_object* x_369; lean_object* x_370; lean_object* x_371; lean_object* x_372; lean_object* x_373; lean_object* x_374; lean_object* x_375; lean_object* x_376; lean_object* x_377; lean_object* x_378; lean_object* x_379; lean_object* x_380; lean_object* x_381; lean_object* x_382; lean_object* x_383; lean_object* x_384; lean_object* x_385; lean_object* x_386; lean_object* x_387; lean_object* x_388; lean_object* x_389; lean_object* x_390; lean_object* x_391; lean_object* x_392; lean_object* x_393; lean_object* x_394; lean_object* x_395; lean_object* x_396; lean_object* x_397; lean_object* x_398; lean_object* x_399; lean_object* x_400; lean_object* x_401; lean_object* x_402; lean_object* x_403; lean_object* x_404; lean_object* x_405; lean_object* x_406; lean_object* x_407; lean_object* x_408; lean_object* x_409; lean_object* x_410; lean_object* x_411; lean_object* x_412; lean_object* x_413; lean_object* x_414; lean_object* x_415; lean_object* x_416; lean_object* x_417; lean_object* x_418; lean_object* x_419; lean_object* x_420; lean_object* x_421; lean_object* x_422; lean_object* x_423; lean_object* x_424; lean_object* x_425; lean_object* x_426; lean_object* x_427; lean_object* x_428; lean_object* x_429; lean_object* x_430; lean_object* x_431; lean_object* x_432; lean_object* x_433; lean_object* x_434; lean_object* x_435; lean_object* x_436; lean_object* x_437; lean_object* x_438; lean_object* x_439; lean_object* x_440; lean_object* x_441; lean_object* x_442; lean_object* x_443; lean_object* x_444; lean_object* x_445; lean_object* x_446; lean_object* x_447; lean_object* x_448; lean_object* x_449; lean_object* x_450; lean_object* x_451; lean_object* x_452; lean_object* x_453; lean_object* x_454; lean_object* x_455; lean_object* x_456; lean_object* x_457; lean_object* x_458; lean_object* x_459; lean_object* x_460; lean_object* x_461; lean_object* x_462; lean_object* x_463; lean_object* x_464; lean_object* x_465; lean_object* x_466; lean_object* x_467; lean_object* x_468; lean_object* x_469; lean_object* x_470; lean_object* x_471; lean_object* x_472; lean_object* x_473; lean_object* x_474; lean_object* x_475; lean_object* x_476; lean_object* x_477; lean_object* x_478; lean_object* x_479; lean_object* x_480; lean_object* x_481; lean_object* x_482; lean_object* x_483; lean_object* x_484; lean_object* x_485; lean_object* x_486; lean_object* x_487; lean_object* x_488; lean_object* x_489; lean_object* x_490; lean_object* x_491; lean_object* x_492; lean_object* x_493; lean_object* x_494; lean_object* x_495; lean_object* x_496; lean_object* x_497; lean_object* x_498; lean_object* x_499; lean_object* x_500; lean_object* x_501; lean_object* x_502; lean_object* x_503; lean_object* x_504; lean_object* x_505; lean_object* x_506; lean_object* x_507; lean_object* x_508; lean_object* x_509; lean_object* x_510; lean_object* x_511; lean_object* x_512; lean_object* x_513; lean_object* x_514; lean_object* x_515; lean_object* x_516; lean_object* x_517; lean_object* x_518; lean_object* x_519; lean_object* x_520; lean_object* x_521; lean_object* x_522; lean_object* x_523; lean_object* x_524; lean_object* x_525; lean_object* x_526; lean_object* x_527; lean_object* x_528; lean_object* x_529; lean_object* x_530; lean_object* x_531; lean_object* x_532; lean_object* x_533; lean_object* x_534; lean_object* x_535; lean_object* x_536; lean_object* x_537; lean_object* x_538; lean_object* x_539; lean_object* x_540; lean_object* x_541; lean_object* x_542; lean_object* x_543; lean_object* x_544; lean_object* x_545; lean_object* x_546; lean_object* x_547; lean_object* x_548; lean_object* x_549; lean_object* x_550; lean_object* x_551; lean_object* x_552; lean_object* x_553; lean_object* x_554; lean_object* x_555; lean_object* x_556; lean_object* x_557; lean_object* x_558; lean_object* x_559; lean_object* x_560; lean_object* x_561; lean_object* x_562; lean_object* x_563; lean_object* x_564; lean_object* x_565; lean_object* x_566; lean_object* x_567; lean_object* x_568; lean_object* x_569; lean_object* x_570; lean_object* x_571; lean_object* x_572; lean_object* x_573; lean_object* x_574; lean_object* x_575; lean_object* x_576; lean_object* x_577; lean_object* x_578; lean_object* x_579; lean_object* x_580; lean_object* x_581; lean_object* x_582; lean_object* x_583; lean_object* x_584; lean_object* x_585; lean_object* x_586; lean_object* x_587; lean_object* x_588; lean_object* x_589; lean_object* x_590; lean_object* x_591; lean_object* x_592; lean_object* x_593; lean_object* x_594; lean_object* x_595; lean_object* x_596; lean_object* x_597; lean_object* x_598; lean_object* x_599; lean_object* x_600; lean_object* x_601; lean_object* x_602; lean_object* x_603; lean_object* x_604; lean_object* x_605; lean_object* x_606; lean_object* x_607; lean_object* x_608; lean_object* x_609; lean_object* x_610; lean_object* x_611; lean_object* x_612; lean_object* x_613; lean_object* x_614; lean_object* x_615; lean_object* x_616; lean_object* x_617; lean_object* x_618; lean_object* x_619; lean_object* x_620; lean_object* x_621; lean_object* x_622; lean_object* x_623; lean_object* x_624; lean_object* x_625; lean_object* x_626; lean_object* x_627; lean_object* x_628; lean_object* x_629; lean_object* x_630; lean_object* x_631; lean_object* x_632; lean_object* x_633; lean_object* x_634; lean_object* x_635; lean_object* x_636; lean_object* x_637; lean_object* x_638; lean_object* x_639; lean_object* x_640; lean_object* x_641; lean_object* x_642; lean_object* x_643; lean_object* x_644; lean_object* x_645; lean_object* x_646; lean_object* x_647; lean_object* x_648; lean_object* x_649; lean_object* x_650; lean_object* x_651; lean_object* x_652; lean_object* x_653; lean_object* x_654; lean_object* x_655; lean_object* x_656; lean_object* x_657; lean_object* x_658; lean_object* x_659; lean_object* x_660; lean_object* x_661; lean_object* x_662; lean_object* x_663; lean_object* x_664; lean_object* x_665; lean_object* x_666; lean_object* x_667; lean_object* x_668; lean_object* x_669; lean_object* x_670; lean_object* x_671; lean_object* x_672; lean_object* x_673; lean_object* x_674; lean_object* x_675; lean_object* x_676; lean_object* x_677; lean_object* x_678; lean_object* x_679; lean_object* x_680; lean_object* x_681; lean_object* x_682; lean_object* x_683; lean_object* x_684; lean_object* x_685; lean_object* x_686; lean_object* x_687; lean_object* x_688; lean_object* x_689; lean_object* x_690; lean_object* x_691; lean_object* x_692; lean_object* x_693; lean_object* x_694; lean_object* x_695; lean_object* x_696; lean_object* x_697; lean_object* x_698; lean_object* x_699; lean_object* x_700; lean_object* x_701; lean_object* x_702; lean_object* x_703; lean_object* x_704; lean_object* x_705; lean_object* x_706; lean_object* x_707; lean_object* x_708; lean_object* x_709; lean_object* x_710; lean_object* x_711; lean_object* x_712; lean_object* x_713; lean_object* x_714; lean_object* x_715; lean_object* x_716; lean_object* x_717; lean_object* x_718; lean_object* x_719; lean_object* x_720; lean_object* x_721; lean_object* x_722; lean_object* x_723; lean_object* x_724; lean_object* x_725; lean_object* x_726; lean_object* x_727; lean_object* x_728; lean_object* x_729; lean_object* x_730; lean_object* x_731; lean_object* x_732; lean_object* x_733; lean_object* x_734; lean_object* x_735; lean_object* x_736; lean_object* x_737; lean_object* x_738; lean_object* x_739; lean_object* x_740; lean_object* x_741; lean_object* x_742; lean_object* x_743; lean_object* x_744; lean_object* x_745; lean_object* x_746; lean_object* x_747; lean_object* x_748; lean_object* x_749; lean_object* x_750; lean_object* x_751; lean_object* x_752; lean_object* x_753; lean_object* x_754; lean_object* x_755; lean_object* x_756; lean_object* x_757; lean_object* x_758; lean_object* x_759; lean_object* x_760; lean_object* x_761; lean_object* x_762; lean_object* x_763; lean_object* x_764; lean_object* x_765; lean_object* x_766; lean_object* x_767; lean_object* x_768; lean_object* x_769; lean_object* x_770; lean_object* x_771; lean_object* x_772; lean_object* x_773; lean_object* x_774; lean_object* x_775; lean_object* x_776; lean_object* x_777; lean_object* x_778; lean_object* x_779; lean_object* x_780; lean_object* x_781; lean_object* x_782; lean_object* x_783; lean_object* x_784; lean_object* x_785; lean_object* x_786; lean_object* x_787; lean_object* x_788; lean_object* x_789; lean_object* x_790; lean_object* x_791; lean_object* x_792; lean_object* x_793; lean_object* x_794; lean_object* x_795; lean_object* x_796; lean_object* x_797; lean_object* x_798; lean_object* x_799; lean_object* x_800; lean_object* x_801; lean_object* x_802; lean_object* x_803; lean_object* x_804; lean_object* x_805; lean_object* x_806; lean_object* x_807; lean_object* x_808; lean_object* x_809; lean_object* x_810; lean_object* x_811; lean_object* x_812; lean_object* x_813; lean_object* x_814; lean_object* x_815; lean_object* x_816; lean_object* x_817; lean_object* x_818; lean_object* x_819; lean_object* x_820; lean_object* x_821; lean_object* x_822; lean_object* x_823; lean_object* x_824; lean_object* x_825; lean_object* x_826; lean_object* x_827; lean_object* x_828; lean_object* x_829; lean_object* x_830; lean_object* x_831; lean_object* x_832; lean_object* x_833; lean_object* x_834; lean_object* x_835; lean_object* x_836; lean_object* x_837; lean_object* x_838; lean_object* x_839; lean_object* x_840; lean_object* x_841; lean_object* x_842; lean_object* x_843; lean_object* x_844; lean_object* x_845; lean_object* x_846; lean_object* x_847; lean_object* x_848; lean_object* x_849; lean_object* x_850; lean_object* x_851; lean_object* x_852; lean_object* x_853; lean_object* x_854; lean_object* x_855; lean_object* x_856; lean_object* x_857; lean_object* x_858; lean_object* x_859; lean_object* x_860; lean_object* x_861; lean_object* x_862; lean_object* x_863; lean_object* x_864; lean_object* x_865; lean_object* x_866; lean_object* x_867; lean_object* x_868; lean_object* x_869; lean_object* x_870; lean_object* x_871; lean_object* x_872; lean_object* x_873; lean_object* x_874; lean_object* x_875; lean_object* x_876; lean_object* x_877; lean_object* x_878; lean_object* x_879; lean_object* x_880; lean_object* x_881; lean_object* x_882; lean_object* x_883; lean_object* x_884; lean_object* x_885; lean_object* x_886; lean_object* x_887; lean_object* x_888; lean_object* x_889; lean_object* x_890; lean_object* x_891; lean_object* x_892; lean_object* x_893; lean_object* x_894; lean_object* x_895; lean_object* x_896; lean_object* x_897; lean_object* x_898; lean_object* x_899; lean_object* x_900; lean_object* x_901; lean_object* x_902; lean_object* x_903; lean_object* x_904; lean_object* x_905; lean_object* x_906; lean_object* x_907; lean_object* x_908; lean_object* x_909; lean_object* x_910; lean_object* x_911; lean_object* x_912; lean_object* x_913; lean_object* x_914; lean_object* x_915; lean_object* x_916; lean_object* x_917; lean_object* x_918; lean_object* x_919; lean_object* x_920; lean_object* x_921; lean_object* x_922; lean_object* x_923; lean_object* x_924; lean_object* x_925; lean_object* x_926; lean_object* x_927; lean_object* x_928; lean_object* x_929; lean_object* x_930; lean_object* x_931; lean_object* x_932; lean_object* x_933; lean_object* x_934; lean_object* x_935; lean_object* x_936; lean_object* x_937; lean_object* x_938; lean_object* x_939; lean_object* x_940; lean_object* x_941; lean_object* x_942; lean_object* x_943; lean_object* x_944; lean_object* x_945; lean_object* x_946; lean_object* x_947; lean_object* x_948; lean_object* x_949; lean_object* x_950; lean_object* x_951; lean_object* x_952; lean_object* x_953; lean_object* x_954; lean_object* x_955; lean_object* x_956; lean_object* x_957; lean_object* x_958; lean_object* x_959; lean_object* x_960; lean_object* x_961; lean_object* x_962; lean_object* x_963; lean_object* x_964; lean_object* x_965; lean_object* x_966; lean_object* x_967; lean_object* x_968; lean_object* x_969; lean_object* x_970; lean_object* x_971; lean_object* x_972; lean_object* x_973; lean_object* x_974; lean_object* x_975; lean_object* x_976; lean_object* x_977; lean_object* x_978; lean_object* x_979; lean_object* x_980; lean_object* x_981; lean_object* x_982; lean_object* x_983; lean_object* x_984; lean_object* x_985; lean_object* x_986; lean_object* x_987; lean_object* x_988; lean_object* x_989; lean_object* x_990; lean_object* x_991; lean_object* x_992; lean_object* x_993; lean_object* x_994; lean_object* x_995; lean_object* x_996; lean_object* x_997; lean_object* x_998; lean_object* x_999; lean_object* x_1000; lean_object* x_1001; lean_object* x_1002; lean_object* x_1003; lean_object* x_1004; lean_object* x_1005; lean_object* x_1006; lean_object* x_1007; lean_object* x_1008; lean_object* x_1009; lean_object* x_1010; lean_object* x_1011; lean_object* x_1012; lean_object* x_1013; lean_object* x_1014; lean_object* x_1015; lean_object* x_1016; lean_object* x_1017; lean_object* x_1018; lean_object* x_1019; lean_object* x_1020; lean_object* x_1021; lean_object* x_1022; lean_object* x_1023; lean_object* x_1024; lean_object* x_1025; lean_object* x_1026; lean_object* x_1027; lean_object* x_1028; lean_object* x_1029; lean_object* x_1030; lean_object* x_1031; lean_object* x_1032; lean_object* x_1033; lean_object* x_1034; lean_object* x_1035; lean_object* x_1036; lean_object* x_1037; lean_object* x_1038; lean_object* x_1039; lean_object* x_1040; lean_object* x_1041; lean_object* x_1042; lean_object* x_1043; lean_object* x_1044; lean_object* x_1045; lean_object* x_1046; lean_object* x_1047; lean_object* x_1048; lean_object* x_1049; lean_object* x_1050; lean_object* x_1051; lean_object* x_1052; lean_object* x_1053; lean_object* x_1054; lean_object* x_1055; lean_object* x_1056; lean_object* x_1057; lean_object* x_1058; lean_object* x_1059; lean_object* x_1060; lean_object* x_1061; lean_object* x_1062; lean_object* x_1063; lean_object* x_1064; lean_object* x_1065; lean_object* x_1066; lean_object* x_1067; lean_object* x_1068; lean_object* x_1069; lean_object* x_1070; lean_object* x_1071; lean_object* x_1072; lean_object* x_1073; lean_object* x_1074; lean_object* x_1075; lean_object* x_1076; lean_object* x_1077; lean_object* x_1078; lean_object* x_1079; lean_object* x_1080; lean_object* x_1081; lean_object* x_1082; lean_object* x_1083; lean_object* x_1084; lean_object* x_1085; lean_object* x_1086; lean_object* x_1087; lean_object* x_1088; lean_object* x_1089; lean_object* x_1090; lean_object* x_1091; lean_object* x_1092; lean_object* x_1093; lean_object* x_1094; lean_object* x_1095; lean_object* x_1096; lean_object* x_1097; lean_object* x_1098; lean_object* x_1099; lean_object* x_1100; lean_object* x_1101; lean_object* x_1102; lean_object* x_1103; lean_object* x_1104; lean_object* x_1105; lean_object* x_1106; lean_object* x_1107; lean_object* x_1108; lean_object* x_1109; lean_object* x_1110; lean_object* x_1111; lean_object* x_1112; lean_object* x_1113; lean_object* x_1114; lean_object* x_1115; lean_object* x_1116; lean_object* x_1117; lean_object* x_1118; lean_object* x_1119; lean_object* x_1120; lean_object* x_1121; lean_object* x_1122; lean_object* x_1123; lean_object* x_1124; lean_object* x_1125; lean_object* x_1126; lean_object* x_1127; lean_object* x_1128; lean_object* x_1129; lean_object* x_1130; lean_object* x_1131; lean_object* x_1132; lean_object* x_1133; lean_object* x_1134; lean_object* x_1135; lean_object* x_1136; lean_object* x_1137; lean_object* x_1138; lean_object* x_1139; lean_object* x_1140; lean_object* x_1141; lean_object* x_1142; lean_object* x_1143; lean_object* x_1144; lean_object* x_1145; lean_object* x_1146; lean_object* x_1147; lean_object* x_1148; lean_object* x_1149; lean_object* x_1150; lean_object* x_1151; lean_object* x_1152; lean_object* x_1153; lean_object* x_1154; lean_object* x_1155; lean_object* x_1156; lean_object* x_1157; lean_object* x_1158; lean_object* x_1159; lean_object* x_1160; lean_object* x_1161; lean_object* x_1162; lean_object* x_1163; lean_object* x_1164; lean_object* x_1165; lean_object* x_1166; lean_object* x_1167; lean_object* x_1168; lean_object* x_1169; lean_object* x_1170; lean_object* x_1171; lean_object* x_1172; lean_object* x_1173; +lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; lean_object* x_286; lean_object* x_287; lean_object* x_288; lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; lean_object* x_294; lean_object* x_295; lean_object* x_296; lean_object* x_297; lean_object* x_298; lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; lean_object* x_307; lean_object* x_308; lean_object* x_309; lean_object* x_310; lean_object* x_311; lean_object* x_312; lean_object* x_313; lean_object* x_314; lean_object* x_315; lean_object* x_316; lean_object* x_317; lean_object* x_318; lean_object* x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; lean_object* x_324; lean_object* x_325; lean_object* x_326; lean_object* x_327; lean_object* x_328; lean_object* x_329; lean_object* x_330; lean_object* x_331; lean_object* x_332; lean_object* x_333; lean_object* x_334; lean_object* x_335; lean_object* x_336; lean_object* x_337; lean_object* x_338; lean_object* x_339; lean_object* x_340; lean_object* x_341; lean_object* x_342; lean_object* x_343; lean_object* x_344; lean_object* x_345; lean_object* x_346; lean_object* x_347; lean_object* x_348; lean_object* x_349; lean_object* x_350; lean_object* x_351; lean_object* x_352; lean_object* x_353; lean_object* x_354; lean_object* x_355; lean_object* x_356; lean_object* x_357; lean_object* x_358; lean_object* x_359; lean_object* x_360; lean_object* x_361; lean_object* x_362; lean_object* x_363; lean_object* x_364; lean_object* x_365; lean_object* x_366; lean_object* x_367; lean_object* x_368; lean_object* x_369; lean_object* x_370; lean_object* x_371; lean_object* x_372; lean_object* x_373; lean_object* x_374; lean_object* x_375; lean_object* x_376; lean_object* x_377; lean_object* x_378; lean_object* x_379; lean_object* x_380; lean_object* x_381; lean_object* x_382; lean_object* x_383; lean_object* x_384; lean_object* x_385; lean_object* x_386; lean_object* x_387; lean_object* x_388; lean_object* x_389; lean_object* x_390; lean_object* x_391; lean_object* x_392; lean_object* x_393; lean_object* x_394; lean_object* x_395; lean_object* x_396; lean_object* x_397; lean_object* x_398; lean_object* x_399; lean_object* x_400; lean_object* x_401; lean_object* x_402; lean_object* x_403; lean_object* x_404; lean_object* x_405; lean_object* x_406; lean_object* x_407; lean_object* x_408; lean_object* x_409; lean_object* x_410; lean_object* x_411; lean_object* x_412; lean_object* x_413; lean_object* x_414; lean_object* x_415; lean_object* x_416; lean_object* x_417; lean_object* x_418; lean_object* x_419; lean_object* x_420; lean_object* x_421; lean_object* x_422; lean_object* x_423; lean_object* x_424; lean_object* x_425; lean_object* x_426; lean_object* x_427; lean_object* x_428; lean_object* x_429; lean_object* x_430; lean_object* x_431; lean_object* x_432; lean_object* x_433; lean_object* x_434; lean_object* x_435; lean_object* x_436; lean_object* x_437; lean_object* x_438; lean_object* x_439; lean_object* x_440; lean_object* x_441; lean_object* x_442; lean_object* x_443; lean_object* x_444; lean_object* x_445; lean_object* x_446; lean_object* x_447; lean_object* x_448; lean_object* x_449; lean_object* x_450; lean_object* x_451; lean_object* x_452; lean_object* x_453; lean_object* x_454; lean_object* x_455; lean_object* x_456; lean_object* x_457; lean_object* x_458; lean_object* x_459; lean_object* x_460; lean_object* x_461; lean_object* x_462; lean_object* x_463; lean_object* x_464; lean_object* x_465; lean_object* x_466; lean_object* x_467; lean_object* x_468; lean_object* x_469; lean_object* x_470; lean_object* x_471; lean_object* x_472; lean_object* x_473; lean_object* x_474; lean_object* x_475; lean_object* x_476; lean_object* x_477; lean_object* x_478; lean_object* x_479; lean_object* x_480; lean_object* x_481; lean_object* x_482; lean_object* x_483; lean_object* x_484; lean_object* x_485; lean_object* x_486; lean_object* x_487; lean_object* x_488; lean_object* x_489; lean_object* x_490; lean_object* x_491; lean_object* x_492; lean_object* x_493; lean_object* x_494; lean_object* x_495; lean_object* x_496; lean_object* x_497; lean_object* x_498; lean_object* x_499; lean_object* x_500; lean_object* x_501; lean_object* x_502; lean_object* x_503; lean_object* x_504; lean_object* x_505; lean_object* x_506; lean_object* x_507; lean_object* x_508; lean_object* x_509; lean_object* x_510; lean_object* x_511; lean_object* x_512; lean_object* x_513; lean_object* x_514; lean_object* x_515; lean_object* x_516; lean_object* x_517; lean_object* x_518; lean_object* x_519; lean_object* x_520; lean_object* x_521; lean_object* x_522; lean_object* x_523; lean_object* x_524; lean_object* x_525; lean_object* x_526; lean_object* x_527; lean_object* x_528; lean_object* x_529; lean_object* x_530; lean_object* x_531; lean_object* x_532; lean_object* x_533; lean_object* x_534; lean_object* x_535; lean_object* x_536; lean_object* x_537; lean_object* x_538; lean_object* x_539; lean_object* x_540; lean_object* x_541; lean_object* x_542; lean_object* x_543; lean_object* x_544; lean_object* x_545; lean_object* x_546; lean_object* x_547; lean_object* x_548; lean_object* x_549; lean_object* x_550; lean_object* x_551; lean_object* x_552; lean_object* x_553; lean_object* x_554; lean_object* x_555; lean_object* x_556; lean_object* x_557; lean_object* x_558; lean_object* x_559; lean_object* x_560; lean_object* x_561; lean_object* x_562; lean_object* x_563; lean_object* x_564; lean_object* x_565; lean_object* x_566; lean_object* x_567; lean_object* x_568; lean_object* x_569; lean_object* x_570; lean_object* x_571; lean_object* x_572; lean_object* x_573; lean_object* x_574; lean_object* x_575; lean_object* x_576; lean_object* x_577; lean_object* x_578; lean_object* x_579; lean_object* x_580; lean_object* x_581; lean_object* x_582; lean_object* x_583; lean_object* x_584; lean_object* x_585; lean_object* x_586; lean_object* x_587; lean_object* x_588; lean_object* x_589; lean_object* x_590; lean_object* x_591; lean_object* x_592; lean_object* x_593; lean_object* x_594; lean_object* x_595; lean_object* x_596; lean_object* x_597; lean_object* x_598; lean_object* x_599; lean_object* x_600; lean_object* x_601; lean_object* x_602; lean_object* x_603; lean_object* x_604; lean_object* x_605; lean_object* x_606; lean_object* x_607; lean_object* x_608; lean_object* x_609; lean_object* x_610; lean_object* x_611; lean_object* x_612; lean_object* x_613; lean_object* x_614; lean_object* x_615; lean_object* x_616; lean_object* x_617; lean_object* x_618; lean_object* x_619; lean_object* x_620; lean_object* x_621; lean_object* x_622; lean_object* x_623; lean_object* x_624; lean_object* x_625; lean_object* x_626; lean_object* x_627; lean_object* x_628; lean_object* x_629; lean_object* x_630; lean_object* x_631; lean_object* x_632; lean_object* x_633; lean_object* x_634; lean_object* x_635; lean_object* x_636; lean_object* x_637; lean_object* x_638; lean_object* x_639; lean_object* x_640; lean_object* x_641; lean_object* x_642; lean_object* x_643; lean_object* x_644; lean_object* x_645; lean_object* x_646; lean_object* x_647; lean_object* x_648; lean_object* x_649; lean_object* x_650; lean_object* x_651; lean_object* x_652; lean_object* x_653; lean_object* x_654; lean_object* x_655; lean_object* x_656; lean_object* x_657; lean_object* x_658; lean_object* x_659; lean_object* x_660; lean_object* x_661; lean_object* x_662; lean_object* x_663; lean_object* x_664; lean_object* x_665; lean_object* x_666; lean_object* x_667; lean_object* x_668; lean_object* x_669; lean_object* x_670; lean_object* x_671; lean_object* x_672; lean_object* x_673; lean_object* x_674; lean_object* x_675; lean_object* x_676; lean_object* x_677; lean_object* x_678; lean_object* x_679; lean_object* x_680; lean_object* x_681; lean_object* x_682; lean_object* x_683; lean_object* x_684; lean_object* x_685; lean_object* x_686; lean_object* x_687; lean_object* x_688; lean_object* x_689; lean_object* x_690; lean_object* x_691; lean_object* x_692; lean_object* x_693; lean_object* x_694; lean_object* x_695; lean_object* x_696; lean_object* x_697; lean_object* x_698; lean_object* x_699; lean_object* x_700; lean_object* x_701; lean_object* x_702; lean_object* x_703; lean_object* x_704; lean_object* x_705; lean_object* x_706; lean_object* x_707; lean_object* x_708; lean_object* x_709; lean_object* x_710; lean_object* x_711; lean_object* x_712; lean_object* x_713; lean_object* x_714; lean_object* x_715; lean_object* x_716; lean_object* x_717; lean_object* x_718; lean_object* x_719; lean_object* x_720; lean_object* x_721; lean_object* x_722; lean_object* x_723; lean_object* x_724; lean_object* x_725; lean_object* x_726; lean_object* x_727; lean_object* x_728; lean_object* x_729; lean_object* x_730; lean_object* x_731; lean_object* x_732; lean_object* x_733; lean_object* x_734; lean_object* x_735; lean_object* x_736; lean_object* x_737; lean_object* x_738; lean_object* x_739; lean_object* x_740; lean_object* x_741; lean_object* x_742; lean_object* x_743; lean_object* x_744; lean_object* x_745; lean_object* x_746; lean_object* x_747; lean_object* x_748; lean_object* x_749; lean_object* x_750; lean_object* x_751; lean_object* x_752; lean_object* x_753; lean_object* x_754; lean_object* x_755; lean_object* x_756; lean_object* x_757; lean_object* x_758; lean_object* x_759; lean_object* x_760; lean_object* x_761; lean_object* x_762; lean_object* x_763; lean_object* x_764; lean_object* x_765; lean_object* x_766; lean_object* x_767; lean_object* x_768; lean_object* x_769; lean_object* x_770; lean_object* x_771; lean_object* x_772; lean_object* x_773; lean_object* x_774; lean_object* x_775; lean_object* x_776; lean_object* x_777; lean_object* x_778; lean_object* x_779; lean_object* x_780; lean_object* x_781; lean_object* x_782; lean_object* x_783; lean_object* x_784; lean_object* x_785; lean_object* x_786; lean_object* x_787; lean_object* x_788; lean_object* x_789; lean_object* x_790; lean_object* x_791; lean_object* x_792; lean_object* x_793; lean_object* x_794; lean_object* x_795; lean_object* x_796; lean_object* x_797; lean_object* x_798; lean_object* x_799; lean_object* x_800; lean_object* x_801; lean_object* x_802; lean_object* x_803; lean_object* x_804; lean_object* x_805; lean_object* x_806; lean_object* x_807; lean_object* x_808; lean_object* x_809; lean_object* x_810; lean_object* x_811; lean_object* x_812; lean_object* x_813; lean_object* x_814; lean_object* x_815; lean_object* x_816; lean_object* x_817; lean_object* x_818; lean_object* x_819; lean_object* x_820; lean_object* x_821; lean_object* x_822; lean_object* x_823; lean_object* x_824; lean_object* x_825; lean_object* x_826; lean_object* x_827; lean_object* x_828; lean_object* x_829; lean_object* x_830; lean_object* x_831; lean_object* x_832; lean_object* x_833; lean_object* x_834; lean_object* x_835; lean_object* x_836; lean_object* x_837; lean_object* x_838; lean_object* x_839; lean_object* x_840; lean_object* x_841; lean_object* x_842; lean_object* x_843; lean_object* x_844; lean_object* x_845; lean_object* x_846; lean_object* x_847; lean_object* x_848; lean_object* x_849; lean_object* x_850; lean_object* x_851; lean_object* x_852; lean_object* x_853; lean_object* x_854; lean_object* x_855; lean_object* x_856; lean_object* x_857; lean_object* x_858; lean_object* x_859; lean_object* x_860; lean_object* x_861; lean_object* x_862; lean_object* x_863; lean_object* x_864; lean_object* x_865; lean_object* x_866; lean_object* x_867; lean_object* x_868; lean_object* x_869; lean_object* x_870; lean_object* x_871; lean_object* x_872; lean_object* x_873; lean_object* x_874; lean_object* x_875; lean_object* x_876; lean_object* x_877; lean_object* x_878; lean_object* x_879; lean_object* x_880; lean_object* x_881; lean_object* x_882; lean_object* x_883; lean_object* x_884; lean_object* x_885; lean_object* x_886; lean_object* x_887; lean_object* x_888; lean_object* x_889; lean_object* x_890; lean_object* x_891; lean_object* x_892; lean_object* x_893; lean_object* x_894; lean_object* x_895; lean_object* x_896; lean_object* x_897; lean_object* x_898; lean_object* x_899; lean_object* x_900; lean_object* x_901; lean_object* x_902; lean_object* x_903; lean_object* x_904; lean_object* x_905; lean_object* x_906; lean_object* x_907; lean_object* x_908; lean_object* x_909; lean_object* x_910; lean_object* x_911; lean_object* x_912; lean_object* x_913; lean_object* x_914; lean_object* x_915; lean_object* x_916; lean_object* x_917; lean_object* x_918; lean_object* x_919; lean_object* x_920; lean_object* x_921; lean_object* x_922; lean_object* x_923; lean_object* x_924; lean_object* x_925; lean_object* x_926; lean_object* x_927; lean_object* x_928; lean_object* x_929; lean_object* x_930; lean_object* x_931; lean_object* x_932; lean_object* x_933; lean_object* x_934; lean_object* x_935; lean_object* x_936; lean_object* x_937; lean_object* x_938; lean_object* x_939; lean_object* x_940; lean_object* x_941; lean_object* x_942; lean_object* x_943; lean_object* x_944; lean_object* x_945; lean_object* x_946; lean_object* x_947; lean_object* x_948; lean_object* x_949; lean_object* x_950; lean_object* x_951; lean_object* x_952; lean_object* x_953; lean_object* x_954; lean_object* x_955; lean_object* x_956; lean_object* x_957; lean_object* x_958; lean_object* x_959; lean_object* x_960; lean_object* x_961; lean_object* x_962; lean_object* x_963; lean_object* x_964; lean_object* x_965; lean_object* x_966; lean_object* x_967; lean_object* x_968; lean_object* x_969; lean_object* x_970; lean_object* x_971; lean_object* x_972; lean_object* x_973; lean_object* x_974; lean_object* x_975; lean_object* x_976; lean_object* x_977; lean_object* x_978; lean_object* x_979; lean_object* x_980; lean_object* x_981; lean_object* x_982; lean_object* x_983; lean_object* x_984; lean_object* x_985; lean_object* x_986; lean_object* x_987; lean_object* x_988; lean_object* x_989; lean_object* x_990; lean_object* x_991; lean_object* x_992; lean_object* x_993; lean_object* x_994; lean_object* x_995; lean_object* x_996; lean_object* x_997; lean_object* x_998; lean_object* x_999; lean_object* x_1000; lean_object* x_1001; lean_object* x_1002; lean_object* x_1003; lean_object* x_1004; lean_object* x_1005; lean_object* x_1006; lean_object* x_1007; lean_object* x_1008; lean_object* x_1009; lean_object* x_1010; lean_object* x_1011; lean_object* x_1012; lean_object* x_1013; lean_object* x_1014; lean_object* x_1015; lean_object* x_1016; lean_object* x_1017; lean_object* x_1018; lean_object* x_1019; lean_object* x_1020; lean_object* x_1021; lean_object* x_1022; lean_object* x_1023; lean_object* x_1024; lean_object* x_1025; lean_object* x_1026; lean_object* x_1027; lean_object* x_1028; lean_object* x_1029; lean_object* x_1030; lean_object* x_1031; lean_object* x_1032; lean_object* x_1033; lean_object* x_1034; lean_object* x_1035; lean_object* x_1036; lean_object* x_1037; lean_object* x_1038; lean_object* x_1039; lean_object* x_1040; lean_object* x_1041; lean_object* x_1042; lean_object* x_1043; lean_object* x_1044; lean_object* x_1045; lean_object* x_1046; lean_object* x_1047; lean_object* x_1048; lean_object* x_1049; lean_object* x_1050; lean_object* x_1051; lean_object* x_1052; lean_object* x_1053; lean_object* x_1054; lean_object* x_1055; lean_object* x_1056; lean_object* x_1057; lean_object* x_1058; lean_object* x_1059; lean_object* x_1060; lean_object* x_1061; lean_object* x_1062; lean_object* x_1063; lean_object* x_1064; lean_object* x_1065; lean_object* x_1066; lean_object* x_1067; lean_object* x_1068; lean_object* x_1069; lean_object* x_1070; lean_object* x_1071; lean_object* x_1072; lean_object* x_1073; lean_object* x_1074; lean_object* x_1075; lean_object* x_1076; lean_object* x_1077; lean_object* x_1078; lean_object* x_1079; lean_object* x_1080; lean_object* x_1081; lean_object* x_1082; lean_object* x_1083; lean_object* x_1084; lean_object* x_1085; lean_object* x_1086; lean_object* x_1087; lean_object* x_1088; lean_object* x_1089; lean_object* x_1090; lean_object* x_1091; lean_object* x_1092; lean_object* x_1093; lean_object* x_1094; lean_object* x_1095; lean_object* x_1096; lean_object* x_1097; lean_object* x_1098; lean_object* x_1099; lean_object* x_1100; lean_object* x_1101; lean_object* x_1102; lean_object* x_1103; lean_object* x_1104; lean_object* x_1105; lean_object* x_1106; lean_object* x_1107; lean_object* x_1108; lean_object* x_1109; lean_object* x_1110; lean_object* x_1111; lean_object* x_1112; lean_object* x_1113; lean_object* x_1114; lean_object* x_1115; lean_object* x_1116; lean_object* x_1117; lean_object* x_1118; lean_object* x_1119; lean_object* x_1120; lean_object* x_1121; lean_object* x_1122; lean_object* x_1123; lean_object* x_1124; lean_object* x_1125; lean_object* x_1126; lean_object* x_1127; lean_object* x_1128; lean_object* x_1129; lean_object* x_1130; lean_object* x_1131; lean_object* x_1132; lean_object* x_1133; lean_object* x_1134; lean_object* x_1135; lean_object* x_1136; lean_object* x_1137; lean_object* x_1138; lean_object* x_1139; lean_object* x_1140; lean_object* x_1141; lean_object* x_1142; lean_object* x_1143; lean_object* x_1144; lean_object* x_1145; lean_object* x_1146; lean_object* x_1147; lean_object* x_1148; lean_object* x_1149; lean_object* x_1150; lean_object* x_1151; lean_object* x_1152; lean_object* x_1153; lean_object* x_1154; lean_object* x_1155; lean_object* x_1156; lean_object* x_1157; lean_object* x_1158; lean_object* x_1159; lean_object* x_1160; lean_object* x_1161; lean_object* x_1162; lean_object* x_1163; lean_object* x_1164; lean_object* x_1165; lean_object* x_1166; lean_object* x_1167; lean_object* x_1168; lean_object* x_1169; lean_object* x_1170; lean_object* x_1171; lean_object* x_1172; lean_object* x_1173; lean_object* x_1174; lean_object* x_1175; lean_object* x_1176; lean_object* x_1177; lean_object* x_1178; lean_object* x_1179; lean_object* x_1180; lean_object* x_1181; lean_object* x_1182; lean_object* x_1183; lean_object* x_1184; lean_object* x_1185; lean_object* x_1186; lean_object* x_1187; lean_object* x_1188; lean_object* x_1189; lean_object* x_1190; lean_object* x_1191; lean_object* x_1192; lean_object* x_1193; lean_object* x_1194; lean_object* x_1195; lean_object* x_1196; lean_object* x_1197; lean_object* x_1198; lean_object* x_1199; lean_object* x_1200; lean_object* x_1201; lean_object* x_1202; lean_object* x_1203; lean_object* x_1204; lean_object* x_1205; lean_object* x_1206; lean_object* x_1207; lean_object* x_1208; lean_object* x_1209; lean_object* x_1210; lean_object* x_1211; lean_object* x_1212; lean_object* x_1213; lean_object* x_1214; lean_object* x_1215; lean_object* x_1216; lean_object* x_1217; lean_object* x_1218; lean_object* x_1219; lean_object* x_1220; lean_object* x_1221; lean_object* x_1222; lean_object* x_1223; lean_object* x_1224; lean_object* x_1225; lean_object* x_1226; lean_object* x_1227; lean_object* x_1228; lean_object* x_1229; x_8 = lean_unsigned_to_nat(1u); x_9 = l_Lean_Syntax_getArg(x_1, x_8); lean_dec(x_1); @@ -5878,6 +6089,7 @@ lean_ctor_set(x_223, 3, x_28); lean_inc(x_135); lean_inc(x_12); x_224 = l_Lean_Syntax_node1(x_12, x_17, x_135); +lean_inc(x_223); lean_inc(x_12); x_225 = l_Lean_Syntax_node2(x_12, x_33, x_223, x_224); lean_inc(x_120); @@ -5951,6 +6163,7 @@ x_251 = l_Lean_Syntax_node1(x_12, x_250, x_249); lean_inc(x_64); lean_inc(x_12); x_252 = l_Lean_Syntax_node4(x_12, x_96, x_64, x_213, x_230, x_251); +lean_inc(x_209); lean_inc(x_12); x_253 = l_Lean_Syntax_node2(x_12, x_61, x_209, x_252); x_254 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__146; @@ -6141,6 +6354,7 @@ lean_inc(x_12); x_317 = l_Lean_Syntax_node5(x_12, x_126, x_71, x_314, x_316, x_19, x_73); lean_inc(x_12); x_318 = l_Lean_Syntax_node2(x_12, x_17, x_310, x_317); +lean_inc(x_309); lean_inc(x_280); lean_inc(x_12); x_319 = l_Lean_Syntax_node2(x_12, x_33, x_280, x_309); @@ -6160,6 +6374,7 @@ lean_inc(x_323); lean_inc(x_285); lean_inc(x_12); x_324 = l_Lean_Syntax_node3(x_12, x_289, x_320, x_285, x_323); +lean_inc(x_308); lean_inc(x_77); lean_inc(x_12); x_325 = l_Lean_Syntax_node3(x_12, x_85, x_324, x_77, x_308); @@ -7078,6 +7293,7 @@ lean_ctor_set(x_640, 0, x_12); lean_ctor_set(x_640, 1, x_638); lean_ctor_set(x_640, 2, x_639); lean_ctor_set(x_640, 3, x_28); +lean_inc(x_640); lean_inc_n(x_19, 2); lean_inc(x_12); x_641 = l_Lean_Syntax_node3(x_12, x_404, x_19, x_19, x_640); @@ -7650,6 +7866,7 @@ lean_inc(x_831); lean_inc(x_12); x_832 = l_Lean_Syntax_node1(x_12, x_17, x_831); lean_inc(x_265); +lean_inc(x_263); lean_inc(x_832); lean_inc(x_259); lean_inc(x_12); @@ -7812,6 +8029,7 @@ lean_ctor_set(x_889, 0, x_12); lean_ctor_set(x_889, 1, x_887); lean_ctor_set(x_889, 2, x_888); lean_ctor_set(x_889, 3, x_28); +lean_inc(x_236); lean_inc(x_12); x_890 = l_Lean_Syntax_node2(x_12, x_17, x_236, x_859); lean_inc(x_889); @@ -8030,6 +8248,8 @@ x_972 = l_Lean_Syntax_node1(x_12, x_971, x_873); lean_inc(x_972); lean_inc(x_12); x_973 = l_Lean_Syntax_node3(x_12, x_169, x_972, x_168, x_972); +lean_inc(x_73); +lean_inc(x_71); lean_inc(x_12); x_974 = l_Lean_Syntax_node3(x_12, x_282, x_71, x_973, x_73); lean_inc_n(x_19, 2); @@ -8459,144 +8679,302 @@ lean_inc(x_12); x_1123 = l_Lean_Syntax_node2(x_12, x_68, x_1122, x_19); lean_inc(x_12); x_1124 = l_Lean_Syntax_node2(x_12, x_33, x_280, x_107); +lean_inc(x_77); lean_inc(x_12); x_1125 = l_Lean_Syntax_node3(x_12, x_85, x_1124, x_77, x_105); +lean_inc(x_27); lean_inc(x_12); x_1126 = l_Lean_Syntax_node2(x_12, x_35, x_27, x_1125); +lean_inc(x_19); lean_inc(x_12); x_1127 = l_Lean_Syntax_node2(x_12, x_37, x_19, x_1126); +lean_inc(x_95); +lean_inc(x_64); lean_inc(x_12); x_1128 = l_Lean_Syntax_node4(x_12, x_96, x_64, x_1123, x_1127, x_95); lean_inc(x_12); x_1129 = l_Lean_Syntax_node2(x_12, x_61, x_391, x_1128); -x_1130 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__503; -lean_inc(x_12); -x_1131 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_1131, 0, x_12); -lean_ctor_set(x_1131, 1, x_1130); -x_1132 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__504; -lean_inc(x_12); -x_1133 = l_Lean_Syntax_node2(x_12, x_1132, x_1131, x_32); -x_1134 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1134, 0, x_1133); -lean_ctor_set(x_1134, 1, x_28); -x_1135 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1135, 0, x_1129); -lean_ctor_set(x_1135, 1, x_1134); -x_1136 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1136, 0, x_1119); -lean_ctor_set(x_1136, 1, x_1135); -x_1137 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1137, 0, x_1101); +x_1130 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__504; +x_1131 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__505; +lean_inc(x_12); +x_1132 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_1132, 0, x_12); +lean_ctor_set(x_1132, 1, x_1130); +lean_ctor_set(x_1132, 2, x_1131); +lean_ctor_set(x_1132, 3, x_28); +lean_inc(x_19); +lean_inc(x_12); +x_1133 = l_Lean_Syntax_node2(x_12, x_68, x_1132, x_19); +lean_inc(x_73); +lean_inc(x_19); +lean_inc(x_309); +lean_inc(x_71); +lean_inc(x_12); +x_1134 = l_Lean_Syntax_node5(x_12, x_126, x_71, x_309, x_263, x_19, x_73); +lean_inc(x_12); +x_1135 = l_Lean_Syntax_node1(x_12, x_17, x_1134); +x_1136 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__508; +lean_inc(x_12); +x_1137 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_1137, 0, x_12); lean_ctor_set(x_1137, 1, x_1136); -x_1138 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1138, 0, x_1074); -lean_ctor_set(x_1138, 1, x_1137); -x_1139 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1139, 0, x_925); -lean_ctor_set(x_1139, 1, x_1138); -x_1140 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1140, 0, x_821); -lean_ctor_set(x_1140, 1, x_1139); -x_1141 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1141, 0, x_808); -lean_ctor_set(x_1141, 1, x_1140); -x_1142 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1142, 0, x_791); -lean_ctor_set(x_1142, 1, x_1141); -x_1143 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1143, 0, x_770); -lean_ctor_set(x_1143, 1, x_1142); -x_1144 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1144, 0, x_747); -lean_ctor_set(x_1144, 1, x_1143); -x_1145 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1145, 0, x_731); -lean_ctor_set(x_1145, 1, x_1144); -x_1146 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1146, 0, x_691); -lean_ctor_set(x_1146, 1, x_1145); -x_1147 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1147, 0, x_653); -lean_ctor_set(x_1147, 1, x_1146); -x_1148 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1148, 0, x_587); -lean_ctor_set(x_1148, 1, x_1147); -x_1149 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1149, 0, x_555); -lean_ctor_set(x_1149, 1, x_1148); -x_1150 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1150, 0, x_536); -lean_ctor_set(x_1150, 1, x_1149); -x_1151 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1151, 0, x_522); -lean_ctor_set(x_1151, 1, x_1150); -x_1152 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1152, 0, x_500); -lean_ctor_set(x_1152, 1, x_1151); -x_1153 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1153, 0, x_484); -lean_ctor_set(x_1153, 1, x_1152); -x_1154 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1154, 0, x_461); -lean_ctor_set(x_1154, 1, x_1153); -x_1155 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1155, 0, x_445); -lean_ctor_set(x_1155, 1, x_1154); -x_1156 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1156, 0, x_428); -lean_ctor_set(x_1156, 1, x_1155); -x_1157 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1157, 0, x_417); -lean_ctor_set(x_1157, 1, x_1156); -x_1158 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1158, 0, x_385); -lean_ctor_set(x_1158, 1, x_1157); -x_1159 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1159, 0, x_374); -lean_ctor_set(x_1159, 1, x_1158); -x_1160 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1160, 0, x_352); -lean_ctor_set(x_1160, 1, x_1159); -x_1161 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1161, 0, x_301); -lean_ctor_set(x_1161, 1, x_1160); -x_1162 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1162, 0, x_253); -lean_ctor_set(x_1162, 1, x_1161); -x_1163 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1163, 0, x_194); -lean_ctor_set(x_1163, 1, x_1162); -x_1164 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1164, 0, x_178); -lean_ctor_set(x_1164, 1, x_1163); -x_1165 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1165, 0, x_162); -lean_ctor_set(x_1165, 1, x_1164); -x_1166 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1166, 0, x_146); -lean_ctor_set(x_1166, 1, x_1165); -x_1167 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1167, 0, x_113); -lean_ctor_set(x_1167, 1, x_1166); -x_1168 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1168, 0, x_98); -lean_ctor_set(x_1168, 1, x_1167); -x_1169 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1169, 0, x_62); -lean_ctor_set(x_1169, 1, x_1168); -x_1170 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1170, 0, x_16); -lean_ctor_set(x_1170, 1, x_1169); -x_1171 = lean_array_mk(x_1170); -x_1172 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_1172, 0, x_12); -lean_ctor_set(x_1172, 1, x_17); -lean_ctor_set(x_1172, 2, x_1171); -x_1173 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_1173, 0, x_1172); -lean_ctor_set(x_1173, 1, x_3); -return x_1173; +x_1138 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__510; +x_1139 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__512; +lean_inc(x_12); +x_1140 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_1140, 0, x_12); +lean_ctor_set(x_1140, 1, x_1138); +lean_ctor_set(x_1140, 2, x_1139); +lean_ctor_set(x_1140, 3, x_28); +lean_inc(x_12); +x_1141 = l_Lean_Syntax_node2(x_12, x_33, x_1140, x_309); +lean_inc(x_73); +lean_inc(x_1141); +lean_inc(x_71); +lean_inc(x_12); +x_1142 = l_Lean_Syntax_node3(x_12, x_282, x_71, x_1141, x_73); +x_1143 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__507; +lean_inc(x_12); +x_1144 = l_Lean_Syntax_node2(x_12, x_1143, x_1137, x_1142); +lean_inc(x_73); +lean_inc(x_71); +lean_inc(x_12); +x_1145 = l_Lean_Syntax_node3(x_12, x_282, x_71, x_1144, x_73); +lean_inc(x_12); +x_1146 = l_Lean_Syntax_node1(x_12, x_17, x_1145); +lean_inc(x_1146); +lean_inc(x_12); +x_1147 = l_Lean_Syntax_node2(x_12, x_33, x_640, x_1146); +lean_inc(x_1141); +lean_inc(x_77); +lean_inc(x_12); +x_1148 = l_Lean_Syntax_node3(x_12, x_85, x_1147, x_77, x_1141); +lean_inc(x_27); +lean_inc(x_12); +x_1149 = l_Lean_Syntax_node2(x_12, x_35, x_27, x_1148); +lean_inc(x_1135); +lean_inc(x_12); +x_1150 = l_Lean_Syntax_node2(x_12, x_37, x_1135, x_1149); +lean_inc(x_95); +lean_inc(x_64); +lean_inc(x_12); +x_1151 = l_Lean_Syntax_node4(x_12, x_96, x_64, x_1133, x_1150, x_95); +lean_inc(x_209); +lean_inc(x_12); +x_1152 = l_Lean_Syntax_node2(x_12, x_61, x_209, x_1151); +x_1153 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__514; +x_1154 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__515; +lean_inc(x_12); +x_1155 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_1155, 0, x_12); +lean_ctor_set(x_1155, 1, x_1153); +lean_ctor_set(x_1155, 2, x_1154); +lean_ctor_set(x_1155, 3, x_28); +lean_inc(x_19); +lean_inc(x_12); +x_1156 = l_Lean_Syntax_node2(x_12, x_68, x_1155, x_19); +x_1157 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__516; +x_1158 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__517; +lean_inc(x_12); +x_1159 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_1159, 0, x_12); +lean_ctor_set(x_1159, 1, x_1157); +lean_ctor_set(x_1159, 2, x_1158); +lean_ctor_set(x_1159, 3, x_28); +lean_inc(x_12); +x_1160 = l_Lean_Syntax_node2(x_12, x_33, x_1159, x_1146); +x_1161 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__519; +x_1162 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__520; +lean_inc(x_12); +x_1163 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_1163, 0, x_12); +lean_ctor_set(x_1163, 1, x_1161); +lean_ctor_set(x_1163, 2, x_1162); +lean_ctor_set(x_1163, 3, x_28); +lean_inc(x_12); +x_1164 = l_Lean_Syntax_node2(x_12, x_17, x_236, x_308); +lean_inc(x_12); +x_1165 = l_Lean_Syntax_node2(x_12, x_33, x_1163, x_1164); +lean_inc(x_1165); +lean_inc(x_77); +lean_inc(x_12); +x_1166 = l_Lean_Syntax_node3(x_12, x_85, x_1160, x_77, x_1165); +lean_inc(x_27); +lean_inc(x_12); +x_1167 = l_Lean_Syntax_node2(x_12, x_35, x_27, x_1166); +lean_inc(x_1135); +lean_inc(x_12); +x_1168 = l_Lean_Syntax_node2(x_12, x_37, x_1135, x_1167); +lean_inc(x_95); +lean_inc(x_64); +lean_inc(x_12); +x_1169 = l_Lean_Syntax_node4(x_12, x_96, x_64, x_1156, x_1168, x_95); +lean_inc(x_209); +lean_inc(x_12); +x_1170 = l_Lean_Syntax_node2(x_12, x_61, x_209, x_1169); +x_1171 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__522; +x_1172 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__523; +lean_inc(x_12); +x_1173 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_1173, 0, x_12); +lean_ctor_set(x_1173, 1, x_1171); +lean_ctor_set(x_1173, 2, x_1172); +lean_ctor_set(x_1173, 3, x_28); +lean_inc(x_12); +x_1174 = l_Lean_Syntax_node2(x_12, x_68, x_1173, x_19); +lean_inc(x_12); +x_1175 = l_Lean_Syntax_node3(x_12, x_282, x_71, x_1165, x_73); +lean_inc(x_12); +x_1176 = l_Lean_Syntax_node1(x_12, x_17, x_1175); +lean_inc(x_12); +x_1177 = l_Lean_Syntax_node2(x_12, x_33, x_223, x_1176); +lean_inc(x_12); +x_1178 = l_Lean_Syntax_node3(x_12, x_85, x_1177, x_77, x_1141); +lean_inc(x_12); +x_1179 = l_Lean_Syntax_node2(x_12, x_35, x_27, x_1178); +lean_inc(x_12); +x_1180 = l_Lean_Syntax_node2(x_12, x_37, x_1135, x_1179); +lean_inc(x_12); +x_1181 = l_Lean_Syntax_node4(x_12, x_96, x_64, x_1174, x_1180, x_95); +lean_inc(x_12); +x_1182 = l_Lean_Syntax_node2(x_12, x_61, x_209, x_1181); +x_1183 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__524; +lean_inc(x_12); +x_1184 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_1184, 0, x_12); +lean_ctor_set(x_1184, 1, x_1183); +x_1185 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__525; +lean_inc(x_12); +x_1186 = l_Lean_Syntax_node2(x_12, x_1185, x_1184, x_32); +x_1187 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1187, 0, x_1186); +lean_ctor_set(x_1187, 1, x_28); +x_1188 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1188, 0, x_1182); +lean_ctor_set(x_1188, 1, x_1187); +x_1189 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1189, 0, x_1170); +lean_ctor_set(x_1189, 1, x_1188); +x_1190 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1190, 0, x_1152); +lean_ctor_set(x_1190, 1, x_1189); +x_1191 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1191, 0, x_1129); +lean_ctor_set(x_1191, 1, x_1190); +x_1192 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1192, 0, x_1119); +lean_ctor_set(x_1192, 1, x_1191); +x_1193 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1193, 0, x_1101); +lean_ctor_set(x_1193, 1, x_1192); +x_1194 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1194, 0, x_1074); +lean_ctor_set(x_1194, 1, x_1193); +x_1195 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1195, 0, x_925); +lean_ctor_set(x_1195, 1, x_1194); +x_1196 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1196, 0, x_821); +lean_ctor_set(x_1196, 1, x_1195); +x_1197 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1197, 0, x_808); +lean_ctor_set(x_1197, 1, x_1196); +x_1198 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1198, 0, x_791); +lean_ctor_set(x_1198, 1, x_1197); +x_1199 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1199, 0, x_770); +lean_ctor_set(x_1199, 1, x_1198); +x_1200 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1200, 0, x_747); +lean_ctor_set(x_1200, 1, x_1199); +x_1201 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1201, 0, x_731); +lean_ctor_set(x_1201, 1, x_1200); +x_1202 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1202, 0, x_691); +lean_ctor_set(x_1202, 1, x_1201); +x_1203 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1203, 0, x_653); +lean_ctor_set(x_1203, 1, x_1202); +x_1204 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1204, 0, x_587); +lean_ctor_set(x_1204, 1, x_1203); +x_1205 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1205, 0, x_555); +lean_ctor_set(x_1205, 1, x_1204); +x_1206 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1206, 0, x_536); +lean_ctor_set(x_1206, 1, x_1205); +x_1207 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1207, 0, x_522); +lean_ctor_set(x_1207, 1, x_1206); +x_1208 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1208, 0, x_500); +lean_ctor_set(x_1208, 1, x_1207); +x_1209 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1209, 0, x_484); +lean_ctor_set(x_1209, 1, x_1208); +x_1210 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1210, 0, x_461); +lean_ctor_set(x_1210, 1, x_1209); +x_1211 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1211, 0, x_445); +lean_ctor_set(x_1211, 1, x_1210); +x_1212 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1212, 0, x_428); +lean_ctor_set(x_1212, 1, x_1211); +x_1213 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1213, 0, x_417); +lean_ctor_set(x_1213, 1, x_1212); +x_1214 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1214, 0, x_385); +lean_ctor_set(x_1214, 1, x_1213); +x_1215 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1215, 0, x_374); +lean_ctor_set(x_1215, 1, x_1214); +x_1216 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1216, 0, x_352); +lean_ctor_set(x_1216, 1, x_1215); +x_1217 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1217, 0, x_301); +lean_ctor_set(x_1217, 1, x_1216); +x_1218 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1218, 0, x_253); +lean_ctor_set(x_1218, 1, x_1217); +x_1219 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1219, 0, x_194); +lean_ctor_set(x_1219, 1, x_1218); +x_1220 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1220, 0, x_178); +lean_ctor_set(x_1220, 1, x_1219); +x_1221 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1221, 0, x_162); +lean_ctor_set(x_1221, 1, x_1220); +x_1222 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1222, 0, x_146); +lean_ctor_set(x_1222, 1, x_1221); +x_1223 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1223, 0, x_113); +lean_ctor_set(x_1223, 1, x_1222); +x_1224 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1224, 0, x_98); +lean_ctor_set(x_1224, 1, x_1223); +x_1225 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1225, 0, x_62); +lean_ctor_set(x_1225, 1, x_1224); +x_1226 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1226, 0, x_16); +lean_ctor_set(x_1226, 1, x_1225); +x_1227 = lean_array_mk(x_1226); +x_1228 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1228, 0, x_12); +lean_ctor_set(x_1228, 1, x_17); +lean_ctor_set(x_1228, 2, x_1227); +x_1229 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1229, 0, x_1228); +lean_ctor_set(x_1229, 1, x_3); +return x_1229; } } } @@ -9702,6 +10080,48 @@ l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorem lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__503); l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__504 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__504(); lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__504); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__505 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__505(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__505); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__506 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__506(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__506); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__507 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__507(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__507); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__508 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__508(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__508); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__509 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__509(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__509); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__510 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__510(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__510); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__511 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__511(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__511); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__512 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__512(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__512); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__513 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__513(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__513); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__514 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__514(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__514); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__515 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__515(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__515); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__516 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__516(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__516); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__517 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__517(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__517); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__518 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__518(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__518); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__519 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__519(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__519); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__520 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__520(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__520); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__521 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__521(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__521); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__522 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__522(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__522); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__523 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__523(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__523); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__524 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__524(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__524); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__525 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__525(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__525); l_UInt8_instInhabited = _init_l_UInt8_instInhabited(); l_UInt16_instInhabited = _init_l_UInt16_instInhabited(); l_UInt32_instInhabited = _init_l_UInt32_instInhabited(); diff --git a/stage0/stdlib/Init/NotationExtra.c b/stage0/stdlib/Init/NotationExtra.c index a056ecb62ac3..c9d8435f5e69 100644 --- a/stage0/stdlib/Init/NotationExtra.c +++ b/stage0/stdlib/Init/NotationExtra.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Init.NotationExtra -// Imports: Init.Data.ToString.Basic Init.Data.Array.Subarray Init.Conv Init.Meta +// Imports: Init.Data.ToString.Basic Init.Data.Array.Subarray Init.Conv Init.Meta Init.While #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -18,7 +18,6 @@ static lean_object* l_Lean_unbracketedExplicitBinders___closed__11; static lean_object* l___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___closed__14; static lean_object* l_termExists___x2c_____closed__4; static lean_object* l_term_u2203___x2c_____closed__6; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5; static lean_object* l_unexpandEqNDRec___closed__2; static lean_object* l_Lean_unbracketedExplicitBinders___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_classAbbrev; @@ -30,8 +29,6 @@ static lean_object* l_term_x7b___x7d___closed__6; LEAN_EXPORT lean_object* l_unexpandMkArray5(lean_object*, lean_object*, lean_object*); static lean_object* l_term___xd7____1___closed__2; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__11; -static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__3; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__15; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__26; static lean_object* l___aux__Init__NotationExtra______macroRules__term_x7b___x7d__1___closed__2; LEAN_EXPORT lean_object* l_unexpandMkArray3___boxed(lean_object*, lean_object*, lean_object*); @@ -44,8 +41,6 @@ static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__ static lean_object* l_Lean_unbracketedExplicitBinders___closed__3; LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__convCalc____1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___closed__8; -static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__10; -LEAN_EXPORT lean_object* l_Lean_Loop_toCtorIdx___boxed(lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__term_x7b___x7d__1___closed__5; LEAN_EXPORT lean_object* l_unexpandEqNDRec(lean_object*, lean_object*, lean_object*); static lean_object* l_termExists___x2c_____closed__7; @@ -97,7 +92,6 @@ LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__term_x7b_ LEAN_EXPORT lean_object* l_termExists___x2c__; static lean_object* l_term___xd7____1___closed__8; static lean_object* l___aux__Init__NotationExtra______macroRules__term_x7b___x7d__1___lambda__1___closed__4; -static lean_object* l_Lean_doElemRepeat____Until_____closed__8; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Command__classAbbrev__1___lambda__3___closed__9; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__13; @@ -109,21 +103,18 @@ static lean_object* l_Lean_calcFirstStep___closed__7; static lean_object* l_Array_foldrMUnsafe_fold___at___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___spec__4___closed__2; static lean_object* l___aux__Init__NotationExtra______macroRules__term_u03a3___x2c____1___closed__2; LEAN_EXPORT lean_object* l_unexpandSigma(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__1; static lean_object* l_term___xd7_x27____1___closed__5; lean_object* l_Lean_Syntax_getId(lean_object*); static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__57; LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___spec__4(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); static lean_object* l_termExists___x2c_____closed__2; static lean_object* l_Lean_calcSteps___closed__4; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__6; LEAN_EXPORT lean_object* l_unexpandMkArray6(lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___closed__1; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__41; static lean_object* l___aux__Init__NotationExtra______macroRules__tacticFunext________1___lambda__2___closed__3; LEAN_EXPORT lean_object* l_unexpandListNil___rarg___boxed(lean_object*, lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__2; lean_object* l_Array_toSubarray___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_unexpandIte___closed__1; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__26; @@ -163,7 +154,6 @@ static lean_object* l___aux__Init__NotationExtra______macroRules__term_x25_x5b__ static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__11; LEAN_EXPORT lean_object* l_Lean_expandExplicitBindersAux___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__term_x7b___x7d__1(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Loop_forIn___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__16; lean_object* l_Lean_Syntax_TSepArray_getElems___rarg(lean_object*); static lean_object* l_Lean_unifConstraint___closed__3; @@ -176,14 +166,11 @@ static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_ static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__48; LEAN_EXPORT lean_object* l_unexpandListCons___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_term_u03a3___x2c_____closed__2; -LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_classAbbrev___closed__20; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__30; LEAN_EXPORT lean_object* l_Lean_unifConstraintElem; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__17; static lean_object* l_unexpandGetElem_x3f___closed__3; static lean_object* l_unexpandGetElem_x3f___closed__2; -static lean_object* l_Lean_doElemRepeat_____closed__1; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__31; static lean_object* l_Lean_unbracketedExplicitBinders___closed__5; static lean_object* l_Lean_cdotTk___closed__1; @@ -203,13 +190,11 @@ static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___spec__4(size_t, size_t, lean_object*); static lean_object* l_Lean_bracketedExplicitBinders___closed__13; LEAN_EXPORT lean_object* l_Lean_expandExplicitBindersAux_loop___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_doElemRepeat____Until_____closed__5; static lean_object* l_term_u03a3_x27___x2c_____closed__4; lean_object* l_Lean_Syntax_node5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_unexpandGetElem_x21(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7; static lean_object* l_Lean_unifConstraintElem___closed__6; static lean_object* l_Lean_Parser_Command_classAbbrev___closed__27; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__40; @@ -220,13 +205,11 @@ static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__com static lean_object* l_Array_foldrMUnsafe_fold___at___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___spec__4___closed__4; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__17; static lean_object* l_term___xd7_x27____1___closed__6; -LEAN_EXPORT lean_object* l_Lean_instForInLoopUnit___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_unexpandListToArray___closed__2; static lean_object* l_tacticFunext_________closed__3; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__27; static lean_object* l___aux__Init__NotationExtra______macroRules__term_x7b___x7d__1___lambda__1___closed__1; static lean_object* l_Lean_unifConstraint___closed__16; -static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__2; static lean_object* l_Lean_Parser_Command_classAbbrev___closed__2; LEAN_EXPORT lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2__; static lean_object* l_Lean_expandExplicitBindersAux_loop___closed__8; @@ -239,7 +222,6 @@ static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__ LEAN_EXPORT lean_object* l_unexpandProdMk___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Term__letI__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__term_x7b___x7d__1___lambda__1___closed__7; -static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__14; static lean_object* l_term___xd7____1___closed__4; static lean_object* l_term_u03a3___x2c_____closed__8; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__12; @@ -247,7 +229,6 @@ static lean_object* l_term_u03a3_x27___x2c_____closed__6; static lean_object* l_Lean_cdotTk___closed__8; static lean_object* l_Lean_explicitBinders___closed__5; static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Command__classAbbrev__1___lambda__3___closed__5; -LEAN_EXPORT lean_object* l_Lean_instForInLoopUnit(lean_object*, lean_object*); static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__1; LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Command__classAbbrev__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Command__classAbbrev__1___lambda__3___closed__7; @@ -266,10 +247,8 @@ static lean_object* l_term_u2203___x2c_____closed__2; LEAN_EXPORT lean_object* l_unexpandExists___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__term___xd7____1__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean___aux__Init__NotationExtra______macroRules__Lean__solveTactic__1___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_doElemRepeat____Until__; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__53; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___spec__3(size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_unexpandExists___closed__3; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__19; static lean_object* l_termExists___x2c_____closed__5; @@ -281,21 +260,17 @@ static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__com static lean_object* l_unexpandExists___closed__1; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__39; static lean_object* l_Array_mapMUnsafe_map___at_Lean___aux__Init__NotationExtra______macroRules__Lean__solveTactic__1___spec__3___closed__1; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__1; static lean_object* l_tacticFunext_________closed__8; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__46; static lean_object* l_Lean_term__Matches___x7c___closed__9; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__46; -lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_sequenceMap___at_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___spec__1___boxed(lean_object*, lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___closed__6; LEAN_EXPORT lean_object* l_unexpandSubtype(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__28; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__9; size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_expandExplicitBinders___spec__1(lean_object*, size_t, size_t); static lean_object* l_Lean_cdotTk___closed__3; -LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1(lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___closed__15; static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Command__classAbbrev__1___lambda__3___closed__1; static lean_object* l_Lean_expandExplicitBindersAux_loop___closed__13; @@ -314,18 +289,13 @@ static lean_object* l_Lean_bracketedExplicitBinders___closed__12; LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__termExists___x2c____1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__28; static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Term__haveI__1___closed__4; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8; -static lean_object* l_Lean_doElemRepeat_____closed__8; static lean_object* l_Lean_Parser_Command_classAbbrev___closed__30; static lean_object* l_Lean_expandExplicitBindersAux_loop___closed__7; static lean_object* l___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___closed__12; static lean_object* l_Lean_calcSteps___closed__12; -static lean_object* l_Lean_doElemRepeat_____closed__2; LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Command__classAbbrev__1___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__11; static lean_object* l_tacticFunext_________closed__6; static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Term__haveI__1___closed__9; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__14; LEAN_EXPORT lean_object* l_Array_sequenceMap_loop___at_Lean___aux__Init__NotationExtra______macroRules__Lean__solveTactic__1___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_sequenceMap_loop___at___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_unexpandSubtype___closed__2; @@ -394,15 +364,12 @@ static lean_object* l_Lean_expandExplicitBindersAux_loop___closed__9; lean_object* l_Lean_Syntax_getKind(lean_object*); static lean_object* l_Lean_unbracketedExplicitBinders___closed__17; static lean_object* l___aux__Init__NotationExtra______macroRules__tacticFunext________1___lambda__2___closed__8; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__16; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__12; static lean_object* l_term_x7b___x7d___closed__8; lean_object* l_Lean_mkCIdentFrom(lean_object*, lean_object*, uint8_t); static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Command__classAbbrev__1___lambda__3___closed__11; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__20; static lean_object* l_Lean_Parser_Command_classAbbrev___closed__10; static lean_object* l_Lean_unifConstraintElem___closed__11; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____Until____1___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___spec__3___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__14; static lean_object* l_unexpandListNil___rarg___closed__3; @@ -414,13 +381,11 @@ LEAN_EXPORT lean_object* l_unexpandUnit___boxed(lean_object*); static lean_object* l_unexpandSubtype___closed__5; lean_object* l_outOfBounds___rarg(lean_object*); static lean_object* l_Lean_calcTactic___closed__2; -LEAN_EXPORT lean_object* l_Lean_Loop_noConfusion___rarg(lean_object*); LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__tacticFunext________1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_unexpandGetElem_x3f(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__solveTactic__1___lambda__1(lean_object*); static lean_object* l_Lean_solveTactic___closed__11; static lean_object* l_Lean_cdot___closed__6; -static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__13; static lean_object* l_term_x7b___x7d___closed__1; static lean_object* l_Lean_bracketedExplicitBinders___closed__2; static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Command__classAbbrev__1___lambda__3___closed__16; @@ -431,7 +396,6 @@ static lean_object* l_Lean_term__Matches___x7c___closed__10; static lean_object* l_Lean_calcSteps___closed__16; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__59; lean_object* l_Lean_Syntax_getOptional_x3f(lean_object*); -static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__8; static lean_object* l_Lean_calcStep___closed__1; static lean_object* l___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___closed__3; lean_object* l_Lean_Syntax_node3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -440,12 +404,8 @@ static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__ static lean_object* l_Array_foldrMUnsafe_fold___at___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___spec__4___closed__7; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__47; LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__9; static lean_object* l_Lean_calcSteps___closed__3; static lean_object* l_Lean_Parser_Command_classAbbrev___closed__22; -LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___rarg___lambda__1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_doElemRepeat____Until_____closed__4; -static lean_object* l_Lean_doElemWhile__Do_____closed__2; LEAN_EXPORT lean_object* l_Lean_insertUnexpander(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_unexpandIte___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__convCalc____1(lean_object*, lean_object*, lean_object*); @@ -459,7 +419,6 @@ static lean_object* l___aux__Init__NotationExtra______macroRules__term_x7b___x7d LEAN_EXPORT lean_object* l_Lean_expandBrackedBindersAux_loop(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_cdot___closed__5; LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__term___xd7_x27____1__1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__4; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__solveTactic__1___closed__2; static lean_object* l_Lean_cdotTk___closed__11; static lean_object* l_unexpandEqNDRec___closed__1; @@ -471,25 +430,19 @@ static lean_object* l_Lean_explicitBinders___closed__6; LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_solveTactic___closed__8; static lean_object* l_Lean_bracketedExplicitBinders___closed__15; -LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____Until____1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_solveTactic___closed__18; LEAN_EXPORT lean_object* l_Lean_calcTactic; LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__tacticFunext________1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____Until____1___closed__1; static lean_object* l_Array_foldrMUnsafe_fold___at___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___spec__4___closed__9; static lean_object* l_Lean_calcSteps___closed__13; static lean_object* l_Lean_unbracketedExplicitBinders___closed__8; -static lean_object* l_Lean_doElemRepeat____Until_____closed__6; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__23; LEAN_EXPORT lean_object* l_unexpandUnit(lean_object*); static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__19; lean_object* l_Lean_addMacroScope(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__9; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__8; LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__2; lean_object* l_Lean_extractMacroScopes(lean_object*); -LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__term_u2203___x2c____1___closed__1; static lean_object* l_term_u03a3___x2c_____closed__5; static lean_object* l_term_u03a3___x2c_____closed__3; @@ -506,7 +459,6 @@ uint8_t lean_name_eq(lean_object*, lean_object*); static lean_object* l_term___xd7____1___closed__3; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l_Lean_expandExplicitBindersAux_loop___closed__16; -static lean_object* l_Lean_doElemWhile__Do_____closed__1; static lean_object* l_Lean_unifConstraintElem___closed__9; static lean_object* l_Lean_calcFirstStep___closed__3; lean_object* l_Lean_Syntax_node2(lean_object*, lean_object*, lean_object*, lean_object*); @@ -519,7 +471,6 @@ static lean_object* l_term___xd7_x27____1___closed__1; lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); static lean_object* l_Lean_unbracketedExplicitBinders___closed__14; static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Term__haveI__1___lambda__1___closed__2; -LEAN_EXPORT lean_object* l_Lean_Loop_noConfusion___rarg___boxed(lean_object*); LEAN_EXPORT lean_object* l_unexpandSubtype___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__tacticFunext________1___closed__6; static lean_object* l_unexpandListNil___rarg___closed__2; @@ -536,7 +487,6 @@ static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_ uint8_t l_Lean_Syntax_isIdent(lean_object*); static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__3; static lean_object* l_Lean_unifConstraintElem___closed__5; -static lean_object* l_Lean_doElemRepeat_____closed__6; static lean_object* l_Lean_solveTactic___closed__12; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__21; static lean_object* l_Lean_term__Matches___x7c___closed__3; @@ -544,7 +494,6 @@ static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___spec__4___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_unexpandMkArray1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_term___xd7_x27____1___closed__2; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__6; static lean_object* l_Lean_bracketedExplicitBinders___closed__17; LEAN_EXPORT lean_object* l_unexpandArrayEmpty___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_cdotTk; @@ -579,17 +528,14 @@ static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_ static lean_object* l___aux__Init__NotationExtra______macroRules__term_x7b___x7d__1___closed__4; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__49; LEAN_EXPORT lean_object* l_Array_sequenceMap_loop___at_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop(lean_object*, lean_object*); static lean_object* l_Array_foldrMUnsafe_fold___at___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___spec__4___closed__3; static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Term__haveI__1___closed__6; static lean_object* l_term___xd7_x27____1___closed__7; static lean_object* l_term_u03a3_x27___x2c_____closed__2; static lean_object* l_Lean_unifConstraint___closed__13; -LEAN_EXPORT lean_object* l_Lean_Loop_noConfusion(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__32; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__7; static lean_object* l_Lean_term__Matches___x7c___closed__6; -static lean_object* l_Lean_doElemRepeat____Until_____closed__7; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__13; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__42; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__19; @@ -610,7 +556,6 @@ static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__com static lean_object* l_Lean_Parser_Command_classAbbrev___closed__9; static lean_object* l_Lean_calcSteps___closed__15; LEAN_EXPORT lean_object* l_term_u2203___x2c__; -static lean_object* l_Lean_doElemRepeat_____closed__5; static lean_object* l_Lean_bracketedExplicitBinders___closed__5; LEAN_EXPORT lean_object* l_Lean_calcSteps; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__50; @@ -647,13 +592,11 @@ static lean_object* l_Lean_Parser_Command_classAbbrev___closed__15; static lean_object* l_Lean_expandExplicitBindersAux_loop___closed__18; static lean_object* l_tacticFunext_________closed__12; static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Command__classAbbrev__1___lambda__3___closed__12; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__23; LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Command__classAbbrev__1___lambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Command__classAbbrev__1___lambda__1___boxed(lean_object*, lean_object*); static lean_object* l_Lean_unifConstraint___closed__14; static lean_object* l_Lean_calcFirstStep___closed__6; -static lean_object* l_Lean_doElemRepeat____Until_____closed__3; LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__term___xd7____1__1(lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__tacticFunext________1___lambda__2___closed__5; static lean_object* l___aux__Init__NotationExtra______macroRules__term_x7b___x7d__1___closed__6; @@ -662,7 +605,6 @@ static lean_object* l_unexpandGetElem_x21___closed__1; static lean_object* l_term_x7b___x7d___closed__2; static lean_object* l_Lean_expandExplicitBindersAux_loop___closed__4; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__6; -static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__4; static lean_object* l_Lean_calc___closed__5; uint8_t lean_nat_dec_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_unexpandListCons(lean_object*, lean_object*, lean_object*); @@ -679,7 +621,6 @@ lean_object* l_Lean_Syntax_SepArray_ofElems(lean_object*, lean_object*); static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__2; uint8_t lean_nat_dec_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_singletonUnexpander___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__6; LEAN_EXPORT lean_object* l_unexpandProdMk(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_calcStep; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__12; @@ -688,11 +629,9 @@ static lean_object* l_term___xd7_x27____1___closed__4; static lean_object* l_Lean_bracketedExplicitBinders___closed__16; LEAN_EXPORT lean_object* l_term___xd7____1; static lean_object* l_unexpandUnit___rarg___closed__1; -static lean_object* l_Lean_doElemRepeat____Until_____closed__2; LEAN_EXPORT lean_object* l_Lean_expandExplicitBinders___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__8; static lean_object* l_Lean_calcStep___closed__6; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__5; static lean_object* l_Lean_unifConstraint___closed__2; LEAN_EXPORT lean_object* l_unexpandEqRec___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_calcStep___closed__4; @@ -700,8 +639,6 @@ lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_unexpandGetElem___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_expandBrackedBindersAux___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Term__haveI__1___closed__8; -LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3; static lean_object* l_unexpandGetElem_x21___closed__2; LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Term__haveI__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_classAbbrev___closed__12; @@ -718,13 +655,10 @@ lean_object* l_Lean_mkSepArray(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_unexpandMkArray0___boxed(lean_object*); static lean_object* l_Lean_cdotTk___closed__5; -LEAN_EXPORT lean_object* l_Lean_instForInLoopUnit___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_bracketedExplicitBinders___closed__18; static lean_object* l_Lean_expandExplicitBindersAux_loop___closed__17; -LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____Until____1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_calcTactic___closed__4; extern lean_object* l_Lean_binderIdent; -static lean_object* l_Lean_doElemWhile__Do_____closed__3; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__convCalc____1___closed__4; LEAN_EXPORT lean_object* l_Lean_expandExplicitBinders(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_cdotTk___closed__4; @@ -740,7 +674,6 @@ LEAN_EXPORT lean_object* l_unexpandUnit___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_unexpandMkArray0___rarg(lean_object*, lean_object*); static lean_object* l_Lean_unifConstraintElem___closed__4; static lean_object* l_unexpandGetElem_x21___closed__3; -static lean_object* l_Lean_doElemWhile__Do_____closed__6; LEAN_EXPORT lean_object* l_unexpandSigma___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_term_u03a3_x27___x2c_____closed__3; static lean_object* l_Lean_expandExplicitBindersAux_loop___closed__5; @@ -752,24 +685,15 @@ lean_object* lean_nat_sub(lean_object*, lean_object*); static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__45; lean_object* l_Array_mkArray1___rarg(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_expandExplicitBinders___spec__1___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___rarg(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__12; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__22; static lean_object* l_Lean_unbracketedExplicitBinders___closed__23; LEAN_EXPORT lean_object* l_Lean_unbracketedExplicitBinders; -static lean_object* l_Lean_doElemWhile__Do_____closed__5; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__49; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__22; -static lean_object* l_Lean_doElemRepeat_____closed__7; -LEAN_EXPORT lean_object* l_Lean_Loop_toCtorIdx(lean_object*); static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__convCalc____1___closed__9; static lean_object* l_Lean_unbracketedExplicitBinders___closed__21; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__10; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__25; -LEAN_EXPORT lean_object* l_Lean_doElemRepeat__; -LEAN_EXPORT lean_object* l_Lean_Loop_forIn___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Term__haveI__1___closed__7; -static lean_object* l_Lean_doElemRepeat_____closed__3; static lean_object* l_Lean_unbracketedExplicitBinders___closed__10; static lean_object* l___aux__Init__NotationExtra______macroRules__tacticFunext________1___lambda__2___closed__9; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__8; @@ -780,7 +704,6 @@ lean_object* l_Array_ofSubarray___rarg(lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean___aux__Init__NotationExtra______macroRules__Lean__solveTactic__1___spec__3___closed__2; static lean_object* l_tacticFunext_________closed__10; static lean_object* l_Lean_Parser_Command_classAbbrev___closed__29; -static lean_object* l_Lean_doElemRepeat____Until_____closed__1; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__48; LEAN_EXPORT lean_object* l_unexpandListNil___rarg(lean_object*, lean_object*); static lean_object* l_Lean_calcFirstStep___closed__11; @@ -788,15 +711,12 @@ LEAN_EXPORT lean_object* l_unexpandGetElem(lean_object*, lean_object*, lean_obje LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__term___xd7_x27____1__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_solveTactic___closed__17; LEAN_EXPORT lean_object* l_Lean_insertUnexpander___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__7; static lean_object* l_unexpandListCons___closed__3; size_t lean_usize_sub(size_t, size_t); static lean_object* l_Lean_unbracketedExplicitBinders___closed__15; lean_object* lean_array_mk(lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__term_u03a3___x2c____1___closed__1; -LEAN_EXPORT lean_object* l_Lean_doElemWhile___x3a__Do__; static lean_object* l_Array_forInUnsafe_loop___at_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___spec__5___closed__1; -LEAN_EXPORT lean_object* l_Lean_Loop_noConfusion___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_unexpandListToArray___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_tacticFunext_________closed__2; static lean_object* l_Lean_calcSteps___closed__9; @@ -807,7 +727,6 @@ LEAN_EXPORT lean_object* l_unexpandListNil___boxed(lean_object*); static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__33; LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__1(lean_object*); static lean_object* l_Lean_bracketedExplicitBinders___closed__6; -static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__5; LEAN_EXPORT lean_object* l_unexpandTSyntax___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__27; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__solveTactic__1___closed__5; @@ -824,7 +743,6 @@ static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__com static lean_object* l___aux__Init__NotationExtra______macroRules__tacticFunext________1___closed__2; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__3; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__9; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1; extern lean_object* l_Lean_instInhabitedSyntax; LEAN_EXPORT lean_object* l_unexpandArrayEmpty___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_expandExplicitBindersAux_loop(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -837,11 +755,9 @@ static lean_object* l_Lean_term__Matches___x7c___closed__1; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__41; LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__term_x7b___x7d__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__term_x7b___x7d__1___lambda__1___closed__2; -static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__9; static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Term__haveI__1___lambda__1___closed__3; static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Command__classAbbrev__1___lambda__3___closed__8; static lean_object* l___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___closed__9; -LEAN_EXPORT lean_object* l_Lean_doElemWhile__Do__; static lean_object* l_Lean_solveTactic___closed__10; LEAN_EXPORT lean_object* l_Array_sequenceMap___at_Lean___aux__Init__NotationExtra______macroRules__Lean__solveTactic__1___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_unifConstraint___closed__11; @@ -850,17 +766,14 @@ static lean_object* l_term_x7b___x7d___closed__5; static lean_object* l_term___xd7____1___closed__1; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__18; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__6; -static lean_object* l_Lean_doElemRepeat_____closed__4; LEAN_EXPORT lean_object* l_unexpandPSigma(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_unbracketedExplicitBinders___closed__9; -static lean_object* l_Lean_doElemRepeat_____closed__9; lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Syntax_SepArray_getElems___spec__1(lean_object*, size_t, size_t, lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__tacticFunext________1___closed__4; lean_object* lean_array_get_size(lean_object*); static lean_object* l_Lean_convCalc_____closed__1; LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__term_u03a3___x2c____1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Command__classAbbrev__1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__7; static lean_object* l_Array_foldrMUnsafe_fold___at___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___spec__4___closed__5; static lean_object* l_unexpandIte___closed__4; static lean_object* l_Lean_unbracketedExplicitBinders___closed__22; @@ -886,10 +799,8 @@ static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__com LEAN_EXPORT lean_object* l_Lean_expandBrackedBinders___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__term_u03a3_x27___x2c____1___closed__2; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__38; -static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__15; static lean_object* l_Lean_solveTactic___closed__6; static lean_object* l_Lean_bracketedExplicitBinders___closed__10; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__3; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__1; LEAN_EXPORT lean_object* l_tacticFunext______; static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Command__classAbbrev__1___lambda__3___closed__13; @@ -899,7 +810,6 @@ static lean_object* l_Lean_term__Matches___x7c___closed__5; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__54; LEAN_EXPORT lean_object* l_unexpandMkArray4(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___spec__7(lean_object*, size_t, size_t, lean_object*); -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__13; LEAN_EXPORT lean_object* l_Lean_cdot; LEAN_EXPORT lean_object* l_unexpandExists(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__45; @@ -914,14 +824,11 @@ static lean_object* l___aux__Init__NotationExtra______macroRules__term_u2203___x static lean_object* l_Lean_term__Matches___x7c___closed__2; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); static lean_object* l_term_u03a3_x27___x2c_____closed__7; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__11; static lean_object* l_unexpandGetElem_x3f___closed__1; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10; LEAN_EXPORT lean_object* l_unexpandMkArray8(lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__term_u03a3_x27___x2c____1___closed__1; static lean_object* l_Lean_cdot___closed__4; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__16; -static lean_object* l_Lean_doElemWhile__Do_____closed__4; static lean_object* l_Lean_unifConstraint___closed__8; static lean_object* l_Lean_solveTactic___closed__4; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__20; @@ -936,7 +843,6 @@ static lean_object* l_Lean_calcSteps___closed__7; static lean_object* l_unexpandPSigma___closed__1; static lean_object* l_Lean_expandExplicitBindersAux_loop___closed__15; static lean_object* l_Lean_Parser_Command_classAbbrev___closed__14; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__4; LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__tacticFunext________1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Command__classAbbrev__1___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_calcSteps___closed__14; @@ -945,7 +851,6 @@ static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__sol static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__29; static lean_object* l_Array_foldrMUnsafe_fold___at___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___spec__4___closed__1; static lean_object* l_Lean_solveTactic___closed__14; -LEAN_EXPORT lean_object* l_Lean_Loop_forIn(lean_object*, lean_object*); static lean_object* l_Lean_bracketedExplicitBinders___closed__8; static lean_object* _init_l_Lean_unbracketedExplicitBinders___closed__1() { _start: @@ -7593,12 +7498,10 @@ if (x_10 == 0) { lean_object* x_11; uint8_t x_12; x_11 = lean_unsigned_to_nat(2u); -lean_inc(x_9); x_12 = l_Lean_Syntax_matchesNull(x_9, x_11); if (x_12 == 0) { lean_object* x_13; lean_object* x_14; -lean_dec(x_9); x_13 = lean_box(0); x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_13); @@ -7607,90 +7510,39 @@ return x_14; } else { -lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; -x_15 = lean_unsigned_to_nat(0u); -x_16 = l_Lean_Syntax_getArg(x_9, x_15); -x_17 = l_Lean_expandExplicitBindersAux_loop___closed__12; -x_18 = l_Lean_Syntax_isOfKind(x_16, x_17); -if (x_18 == 0) -{ -lean_object* x_19; lean_object* x_20; -lean_dec(x_9); -x_19 = lean_box(0); -x_20 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_20, 0, x_19); -lean_ctor_set(x_20, 1, x_3); -return x_20; -} -else -{ -lean_object* x_21; uint8_t x_22; -x_21 = l_Lean_Syntax_getArg(x_9, x_8); -lean_dec(x_9); -x_22 = l_Lean_Syntax_isOfKind(x_21, x_17); -if (x_22 == 0) -{ -lean_object* x_23; lean_object* x_24; -x_23 = lean_box(0); -x_24 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_24, 0, x_23); -lean_ctor_set(x_24, 1, x_3); -return x_24; -} -else -{ -uint8_t x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_25 = 0; -x_26 = l_Lean_SourceInfo_fromRef(x_2, x_25); -x_27 = l_unexpandSorryAx___closed__1; -lean_inc(x_26); -x_28 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_28, 0, x_26); -lean_ctor_set(x_28, 1, x_27); -x_29 = l_unexpandSorryAx___closed__2; -x_30 = l_Lean_Syntax_node1(x_26, x_29, x_28); -x_31 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_31, 0, x_30); -lean_ctor_set(x_31, 1, x_3); -return x_31; -} -} +uint8_t x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_15 = 0; +x_16 = l_Lean_SourceInfo_fromRef(x_2, x_15); +x_17 = l_unexpandSorryAx___closed__1; +lean_inc(x_16); +x_18 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_18, 0, x_16); +lean_ctor_set(x_18, 1, x_17); +x_19 = l_unexpandSorryAx___closed__2; +x_20 = l_Lean_Syntax_node1(x_16, x_19, x_18); +x_21 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_21, 0, x_20); +lean_ctor_set(x_21, 1, x_3); +return x_21; } } else { -lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; -x_32 = lean_unsigned_to_nat(0u); -x_33 = l_Lean_Syntax_getArg(x_9, x_32); +uint8_t x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_dec(x_9); -x_34 = l_Lean_expandExplicitBindersAux_loop___closed__12; -x_35 = l_Lean_Syntax_isOfKind(x_33, x_34); -if (x_35 == 0) -{ -lean_object* x_36; lean_object* x_37; -x_36 = lean_box(0); -x_37 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_37, 0, x_36); -lean_ctor_set(x_37, 1, x_3); -return x_37; -} -else -{ -uint8_t x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_38 = 0; -x_39 = l_Lean_SourceInfo_fromRef(x_2, x_38); -x_40 = l_unexpandSorryAx___closed__1; -lean_inc(x_39); -x_41 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_41, 0, x_39); -lean_ctor_set(x_41, 1, x_40); -x_42 = l_unexpandSorryAx___closed__2; -x_43 = l_Lean_Syntax_node1(x_39, x_42, x_41); -x_44 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_44, 0, x_43); -lean_ctor_set(x_44, 1, x_3); -return x_44; -} +x_22 = 0; +x_23 = l_Lean_SourceInfo_fromRef(x_2, x_22); +x_24 = l_unexpandSorryAx___closed__1; +lean_inc(x_23); +x_25 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +x_26 = l_unexpandSorryAx___closed__2; +x_27 = l_Lean_Syntax_node1(x_23, x_26, x_25); +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_3); +return x_28; } } } @@ -15456,1555 +15308,224 @@ lean_dec(x_2); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Loop_toCtorIdx(lean_object* x_1) { +static lean_object* _init_l_Lean_term__Matches___x7c___closed__1() { _start: { -lean_object* x_2; -x_2 = lean_unsigned_to_nat(0u); -return x_2; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("term_Matches_|", 14, 14); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Loop_toCtorIdx___boxed(lean_object* x_1) { +static lean_object* _init_l_Lean_term__Matches___x7c___closed__2() { _start: { -lean_object* x_2; -x_2 = l_Lean_Loop_toCtorIdx(x_1); -lean_dec(x_1); -return x_2; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_unbracketedExplicitBinders___closed__1; +x_2 = l_Lean_term__Matches___x7c___closed__1; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Loop_noConfusion___rarg(lean_object* x_1) { +static lean_object* _init_l_Lean_term__Matches___x7c___closed__3() { _start: { -lean_inc(x_1); +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" matches ", 9, 9); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Loop_noConfusion(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +static lean_object* _init_l_Lean_term__Matches___x7c___closed__4() { _start: { -lean_object* x_5; -x_5 = lean_alloc_closure((void*)(l_Lean_Loop_noConfusion___rarg___boxed), 1, 0); -return x_5; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_term__Matches___x7c___closed__3; +x_2 = lean_alloc_ctor(5, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Loop_noConfusion___rarg___boxed(lean_object* x_1) { +static lean_object* _init_l_Lean_term__Matches___x7c___closed__5() { _start: { -lean_object* x_2; -x_2 = l_Lean_Loop_noConfusion___rarg(x_1); -lean_dec(x_1); -return x_2; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_unbracketedExplicitBinders___closed__18; +x_2 = lean_unsigned_to_nat(51u); +x_3 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Loop_noConfusion___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +static lean_object* _init_l_Lean_term__Matches___x7c___closed__6() { _start: { -lean_object* x_5; -x_5 = l_Lean_Loop_noConfusion(x_1, x_2, x_3, x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_5; +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" | ", 3, 3); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +static lean_object* _init_l_Lean_term__Matches___x7c___closed__7() { _start: { -if (lean_obj_tag(x_3) == 0) -{ -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -lean_dec(x_2); -x_4 = lean_ctor_get(x_3, 0); -lean_inc(x_4); -lean_dec(x_3); -x_5 = lean_ctor_get(x_1, 0); -lean_inc(x_5); -lean_dec(x_1); -x_6 = lean_ctor_get(x_5, 1); -lean_inc(x_6); -lean_dec(x_5); -x_7 = lean_apply_2(x_6, lean_box(0), x_4); -return x_7; -} -else -{ -lean_object* x_8; lean_object* x_9; -x_8 = lean_ctor_get(x_3, 0); -lean_inc(x_8); -lean_dec(x_3); -x_9 = l_Lean_Loop_forIn_loop___rarg(x_1, x_2, x_8); -return x_9; -} +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_term__Matches___x7c___closed__6; +x_2 = lean_alloc_ctor(5, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +static lean_object* _init_l_Lean_term__Matches___x7c___closed__8() { _start: { -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_4 = lean_ctor_get(x_1, 1); -lean_inc(x_4); -x_5 = lean_box(0); -lean_inc(x_2); -x_6 = lean_apply_2(x_2, x_5, x_3); -x_7 = lean_alloc_closure((void*)(l_Lean_Loop_forIn_loop___rarg___lambda__1), 3, 2); -lean_closure_set(x_7, 0, x_1); -lean_closure_set(x_7, 1, x_2); -x_8 = lean_apply_4(x_4, lean_box(0), lean_box(0), x_6, x_7); -return x_8; +lean_object* x_1; lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; +x_1 = l_Lean_term__Matches___x7c___closed__5; +x_2 = l_Lean_term__Matches___x7c___closed__6; +x_3 = l_Lean_term__Matches___x7c___closed__7; +x_4 = 0; +x_5 = lean_alloc_ctor(11, 3, 1); +lean_ctor_set(x_5, 0, x_1); +lean_ctor_set(x_5, 1, x_2); +lean_ctor_set(x_5, 2, x_3); +lean_ctor_set_uint8(x_5, sizeof(void*)*3, x_4); +return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop(lean_object* x_1, lean_object* x_2) { +static lean_object* _init_l_Lean_term__Matches___x7c___closed__9() { _start: { -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Lean_Loop_forIn_loop___rarg), 3, 0); -return x_3; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_unbracketedExplicitBinders___closed__5; +x_2 = l_Lean_term__Matches___x7c___closed__4; +x_3 = l_Lean_term__Matches___x7c___closed__8; +x_4 = lean_alloc_ctor(2, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Loop_forIn___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +static lean_object* _init_l_Lean_term__Matches___x7c___closed__10() { _start: { -lean_object* x_5; -x_5 = l_Lean_Loop_forIn_loop___rarg(x_1, x_4, x_3); +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_term__Matches___x7c___closed__2; +x_2 = lean_unsigned_to_nat(50u); +x_3 = lean_unsigned_to_nat(51u); +x_4 = l_Lean_term__Matches___x7c___closed__9; +x_5 = lean_alloc_ctor(4, 4, 0); +lean_ctor_set(x_5, 0, x_1); +lean_ctor_set(x_5, 1, x_2); +lean_ctor_set(x_5, 2, x_3); +lean_ctor_set(x_5, 3, x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Loop_forIn(lean_object* x_1, lean_object* x_2) { +static lean_object* _init_l_Lean_term__Matches___x7c() { _start: { -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Lean_Loop_forIn___rarg___boxed), 4, 0); -return x_3; +lean_object* x_1; +x_1 = l_Lean_term__Matches___x7c___closed__10; +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Loop_forIn___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___spec__1(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { _start: { -lean_object* x_5; -x_5 = l_Lean_Loop_forIn___rarg(x_1, x_2, x_3, x_4); +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ lean_dec(x_2); +lean_dec(x_1); return x_5; } -} -LEAN_EXPORT lean_object* l_Lean_instForInLoopUnit___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: +else { -lean_object* x_5; -x_5 = l_Lean_Loop_forIn_loop___rarg(x_1, x_4, x_3); -return x_5; -} +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; size_t x_11; size_t x_12; lean_object* x_13; +x_7 = lean_array_uget(x_5, x_4); +x_8 = lean_unsigned_to_nat(0u); +x_9 = lean_array_uset(x_5, x_4, x_8); +lean_inc(x_2); +lean_inc(x_1); +x_10 = l_Lean_Syntax_node1(x_1, x_2, x_7); +x_11 = 1; +x_12 = lean_usize_add(x_4, x_11); +x_13 = lean_array_uset(x_9, x_4, x_10); +x_4 = x_12; +x_5 = x_13; +goto _start; } -LEAN_EXPORT lean_object* l_Lean_instForInLoopUnit(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Lean_instForInLoopUnit___rarg___boxed), 4, 0); -return x_3; } } -LEAN_EXPORT lean_object* l_Lean_instForInLoopUnit___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__1() { _start: { -lean_object* x_5; -x_5 = l_Lean_instForInLoopUnit___rarg(x_1, x_2, x_3, x_4); -lean_dec(x_2); +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_unbracketedExplicitBinders___closed__1; +x_2 = l_Lean_expandExplicitBindersAux_loop___closed__1; +x_3 = l_Lean_expandExplicitBindersAux_loop___closed__2; +x_4 = l___aux__Init__NotationExtra______macroRules__tacticFunext________1___closed__5; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_doElemRepeat_____closed__1() { +static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__2() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("doElemRepeat_", 13, 13); +x_1 = lean_mk_string_unchecked("match", 5, 5); return x_1; } } -static lean_object* _init_l_Lean_doElemRepeat_____closed__2() { +static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__3() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_unbracketedExplicitBinders___closed__1; -x_2 = l_Lean_doElemRepeat_____closed__1; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; +x_2 = l_Lean_expandExplicitBindersAux_loop___closed__1; +x_3 = l_Lean_expandExplicitBindersAux_loop___closed__2; +x_4 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__2; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; } } -static lean_object* _init_l_Lean_doElemRepeat_____closed__3() { +static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__4() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("repeat ", 7, 7); +x_1 = lean_mk_string_unchecked("matchDiscr", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_doElemRepeat_____closed__4() { +static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__5() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_doElemRepeat_____closed__3; -x_2 = lean_alloc_ctor(5, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_unbracketedExplicitBinders___closed__1; +x_2 = l_Lean_expandExplicitBindersAux_loop___closed__1; +x_3 = l_Lean_expandExplicitBindersAux_loop___closed__2; +x_4 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__4; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; } } -static lean_object* _init_l_Lean_doElemRepeat_____closed__5() { +static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__6() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("doSeq", 5, 5); +x_1 = lean_mk_string_unchecked("with", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_doElemRepeat_____closed__6() { +static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__7() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_doElemRepeat_____closed__5; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("matchAlts", 9, 9); +return x_1; } } -static lean_object* _init_l_Lean_doElemRepeat_____closed__7() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_doElemRepeat_____closed__6; -x_2 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_doElemRepeat_____closed__8() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_unbracketedExplicitBinders___closed__5; -x_2 = l_Lean_doElemRepeat_____closed__4; -x_3 = l_Lean_doElemRepeat_____closed__7; -x_4 = lean_alloc_ctor(2, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; -} -} -static lean_object* _init_l_Lean_doElemRepeat_____closed__9() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_doElemRepeat_____closed__2; -x_2 = lean_unsigned_to_nat(1022u); -x_3 = l_Lean_doElemRepeat_____closed__8; -x_4 = lean_alloc_ctor(3, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; -} -} -static lean_object* _init_l_Lean_doElemRepeat__() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_doElemRepeat_____closed__9; -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("doFor", 5, 5); -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_unbracketedExplicitBinders___closed__1; -x_2 = l_Lean_expandExplicitBindersAux_loop___closed__1; -x_3 = l_Lean_expandExplicitBindersAux_loop___closed__2; -x_4 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__1; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("for", 3, 3); -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("doForDecl", 9, 9); -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_unbracketedExplicitBinders___closed__1; -x_2 = l_Lean_expandExplicitBindersAux_loop___closed__1; -x_3 = l_Lean_expandExplicitBindersAux_loop___closed__2; -x_4 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__4; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__6() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("in", 2, 2); -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__7() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Loop.mk", 7, 7); -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__8() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__7; -x_2 = l_String_toSubstring_x27(x_1); -return x_2; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__9() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Loop", 4, 4); -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__10() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__9; -x_2 = l___aux__Init__NotationExtra______macroRules__Lean__Parser__Command__classAbbrev__1___lambda__3___closed__15; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__11() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_unbracketedExplicitBinders___closed__1; -x_2 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__9; -x_3 = l___aux__Init__NotationExtra______macroRules__Lean__Parser__Command__classAbbrev__1___lambda__3___closed__15; -x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); -return x_4; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__12() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__11; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__13() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__11; -x_2 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__14() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__13; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__15() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__13; -x_2 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__14; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__16() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__12; -x_2 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__15; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__17() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("do", 2, 2); -return x_1; -} -} -LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; uint8_t x_5; -x_4 = l_Lean_doElemRepeat_____closed__2; -lean_inc(x_1); -x_5 = l_Lean_Syntax_isOfKind(x_1, x_4); -if (x_5 == 0) -{ -lean_object* x_6; lean_object* x_7; -lean_dec(x_2); -lean_dec(x_1); -x_6 = lean_box(1); -x_7 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_7, 0, x_6); -lean_ctor_set(x_7, 1, x_3); -return x_7; -} -else -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_8 = lean_unsigned_to_nat(1u); -x_9 = l_Lean_Syntax_getArg(x_1, x_8); -lean_dec(x_1); -x_10 = lean_ctor_get(x_2, 5); -lean_inc(x_10); -x_11 = 0; -x_12 = l_Lean_SourceInfo_fromRef(x_10, x_11); -lean_dec(x_10); -x_13 = lean_ctor_get(x_2, 2); -lean_inc(x_13); -x_14 = lean_ctor_get(x_2, 1); -lean_inc(x_14); -lean_dec(x_2); -x_15 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__3; -lean_inc(x_12); -x_16 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_16, 0, x_12); -lean_ctor_set(x_16, 1, x_15); -x_17 = l_Lean_expandExplicitBindersAux_loop___closed__6; -x_18 = l_Lean_expandExplicitBindersAux_loop___closed__14; -lean_inc(x_12); -x_19 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_19, 0, x_12); -lean_ctor_set(x_19, 1, x_17); -lean_ctor_set(x_19, 2, x_18); -x_20 = l_Lean_expandExplicitBindersAux_loop___closed__13; -lean_inc(x_12); -x_21 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_21, 0, x_12); -lean_ctor_set(x_21, 1, x_20); -x_22 = l_Lean_expandExplicitBindersAux_loop___closed__12; -lean_inc(x_12); -x_23 = l_Lean_Syntax_node1(x_12, x_22, x_21); -x_24 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__6; -lean_inc(x_12); -x_25 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_25, 0, x_12); -lean_ctor_set(x_25, 1, x_24); -x_26 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__10; -x_27 = l_Lean_addMacroScope(x_14, x_26, x_13); -x_28 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__8; -x_29 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__16; -lean_inc(x_12); -x_30 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_30, 0, x_12); -lean_ctor_set(x_30, 1, x_28); -lean_ctor_set(x_30, 2, x_27); -lean_ctor_set(x_30, 3, x_29); -x_31 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__5; -lean_inc(x_12); -x_32 = l_Lean_Syntax_node4(x_12, x_31, x_19, x_23, x_25, x_30); -lean_inc(x_12); -x_33 = l_Lean_Syntax_node1(x_12, x_17, x_32); -x_34 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__17; -lean_inc(x_12); -x_35 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_35, 0, x_12); -lean_ctor_set(x_35, 1, x_34); -x_36 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__2; -x_37 = l_Lean_Syntax_node4(x_12, x_36, x_16, x_33, x_35, x_9); -x_38 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_38, 0, x_37); -lean_ctor_set(x_38, 1, x_3); -return x_38; -} -} -} -static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("doElemWhile_:_Do_", 17, 17); -return x_1; -} -} -static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_unbracketedExplicitBinders___closed__1; -x_2 = l_Lean_doElemWhile___x3a__Do_____closed__1; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("while ", 6, 6); -return x_1; -} -} -static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_doElemWhile___x3a__Do_____closed__3; -x_2 = lean_alloc_ctor(5, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_unbracketedExplicitBinders___closed__5; -x_2 = l_Lean_doElemWhile___x3a__Do_____closed__4; -x_3 = l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__16; -x_4 = lean_alloc_ctor(2, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; -} -} -static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_unbracketedExplicitBinders___closed__5; -x_2 = l_Lean_doElemWhile___x3a__Do_____closed__5; -x_3 = l_Lean_unbracketedExplicitBinders___closed__16; -x_4 = lean_alloc_ctor(2, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; -} -} -static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__7() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("termBeforeDo", 12, 12); -return x_1; -} -} -static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__8() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_doElemWhile___x3a__Do_____closed__7; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__9() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_doElemWhile___x3a__Do_____closed__8; -x_2 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__10() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_unbracketedExplicitBinders___closed__5; -x_2 = l_Lean_doElemWhile___x3a__Do_____closed__6; -x_3 = l_Lean_doElemWhile___x3a__Do_____closed__9; -x_4 = lean_alloc_ctor(2, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; -} -} -static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__11() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked(" do ", 4, 4); -return x_1; -} -} -static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__12() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_doElemWhile___x3a__Do_____closed__11; -x_2 = lean_alloc_ctor(5, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__13() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_unbracketedExplicitBinders___closed__5; -x_2 = l_Lean_doElemWhile___x3a__Do_____closed__10; -x_3 = l_Lean_doElemWhile___x3a__Do_____closed__12; -x_4 = lean_alloc_ctor(2, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; -} -} -static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__14() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_unbracketedExplicitBinders___closed__5; -x_2 = l_Lean_doElemWhile___x3a__Do_____closed__13; -x_3 = l_Lean_doElemRepeat_____closed__7; -x_4 = lean_alloc_ctor(2, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; -} -} -static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__15() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_doElemWhile___x3a__Do_____closed__2; -x_2 = lean_unsigned_to_nat(1022u); -x_3 = l_Lean_doElemWhile___x3a__Do_____closed__14; -x_4 = lean_alloc_ctor(3, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; -} -} -static lean_object* _init_l_Lean_doElemWhile___x3a__Do__() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_doElemWhile___x3a__Do_____closed__15; -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("doSeqIndent", 11, 11); -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_unbracketedExplicitBinders___closed__1; -x_2 = l_Lean_expandExplicitBindersAux_loop___closed__1; -x_3 = l_Lean_expandExplicitBindersAux_loop___closed__2; -x_4 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("doSeqItem", 9, 9); -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_unbracketedExplicitBinders___closed__1; -x_2 = l_Lean_expandExplicitBindersAux_loop___closed__1; -x_3 = l_Lean_expandExplicitBindersAux_loop___closed__2; -x_4 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("doIf", 4, 4); -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_unbracketedExplicitBinders___closed__1; -x_2 = l_Lean_expandExplicitBindersAux_loop___closed__1; -x_3 = l_Lean_expandExplicitBindersAux_loop___closed__2; -x_4 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("doIfProp", 8, 8); -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_unbracketedExplicitBinders___closed__1; -x_2 = l_Lean_expandExplicitBindersAux_loop___closed__1; -x_3 = l_Lean_expandExplicitBindersAux_loop___closed__2; -x_4 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__9() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("doBreak", 7, 7); -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_unbracketedExplicitBinders___closed__1; -x_2 = l_Lean_expandExplicitBindersAux_loop___closed__1; -x_3 = l_Lean_expandExplicitBindersAux_loop___closed__2; -x_4 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__9; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("break", 5, 5); -return x_1; -} -} -LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; uint8_t x_5; -x_4 = l_Lean_doElemWhile___x3a__Do_____closed__2; -lean_inc(x_1); -x_5 = l_Lean_Syntax_isOfKind(x_1, x_4); -if (x_5 == 0) -{ -lean_object* x_6; lean_object* x_7; -lean_dec(x_1); -x_6 = lean_box(1); -x_7 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_7, 0, x_6); -lean_ctor_set(x_7, 1, x_3); -return x_7; -} -else -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_8 = lean_unsigned_to_nat(1u); -x_9 = l_Lean_Syntax_getArg(x_1, x_8); -x_10 = lean_unsigned_to_nat(3u); -x_11 = l_Lean_Syntax_getArg(x_1, x_10); -x_12 = lean_unsigned_to_nat(5u); -x_13 = l_Lean_Syntax_getArg(x_1, x_12); -lean_dec(x_1); -x_14 = lean_ctor_get(x_2, 5); -x_15 = 0; -x_16 = l_Lean_SourceInfo_fromRef(x_14, x_15); -x_17 = l___aux__Init__NotationExtra______macroRules__tacticFunext________1___closed__4; -lean_inc(x_16); -x_18 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_18, 0, x_16); -lean_ctor_set(x_18, 1, x_17); -x_19 = l_unexpandIte___closed__3; -lean_inc(x_16); -x_20 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_20, 0, x_16); -lean_ctor_set(x_20, 1, x_19); -x_21 = l_Lean_expandExplicitBindersAux_loop___closed__18; -lean_inc(x_16); -x_22 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_22, 0, x_16); -lean_ctor_set(x_22, 1, x_21); -x_23 = l_Lean_expandExplicitBindersAux_loop___closed__6; -lean_inc(x_16); -x_24 = l_Lean_Syntax_node2(x_16, x_23, x_9, x_22); -x_25 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8; -lean_inc(x_16); -x_26 = l_Lean_Syntax_node2(x_16, x_25, x_24, x_11); -x_27 = l_unexpandIte___closed__4; -lean_inc(x_16); -x_28 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_28, 0, x_16); -lean_ctor_set(x_28, 1, x_27); -x_29 = l_Lean_expandExplicitBindersAux_loop___closed__14; -lean_inc(x_16); -x_30 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_30, 0, x_16); -lean_ctor_set(x_30, 1, x_23); -lean_ctor_set(x_30, 2, x_29); -x_31 = l_unexpandIte___closed__5; -lean_inc(x_16); -x_32 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_32, 0, x_16); -lean_ctor_set(x_32, 1, x_31); -x_33 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11; -lean_inc(x_16); -x_34 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_34, 0, x_16); -lean_ctor_set(x_34, 1, x_33); -x_35 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10; -lean_inc(x_16); -x_36 = l_Lean_Syntax_node1(x_16, x_35, x_34); -x_37 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__4; -lean_inc(x_30); -lean_inc(x_16); -x_38 = l_Lean_Syntax_node2(x_16, x_37, x_36, x_30); -lean_inc(x_16); -x_39 = l_Lean_Syntax_node1(x_16, x_23, x_38); -x_40 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__2; -lean_inc(x_16); -x_41 = l_Lean_Syntax_node1(x_16, x_40, x_39); -lean_inc(x_16); -x_42 = l_Lean_Syntax_node2(x_16, x_23, x_32, x_41); -x_43 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__6; -lean_inc(x_30); -lean_inc(x_16); -x_44 = l_Lean_Syntax_node6(x_16, x_43, x_20, x_26, x_28, x_13, x_30, x_42); -lean_inc(x_16); -x_45 = l_Lean_Syntax_node2(x_16, x_37, x_44, x_30); -lean_inc(x_16); -x_46 = l_Lean_Syntax_node1(x_16, x_23, x_45); -lean_inc(x_16); -x_47 = l_Lean_Syntax_node1(x_16, x_40, x_46); -x_48 = l_Lean_doElemRepeat_____closed__2; -x_49 = l_Lean_Syntax_node2(x_16, x_48, x_18, x_47); -x_50 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_50, 0, x_49); -lean_ctor_set(x_50, 1, x_3); -return x_50; -} -} -} -LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1(x_1, x_2, x_3); -lean_dec(x_2); -return x_4; -} -} -static lean_object* _init_l_Lean_doElemWhile__Do_____closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("doElemWhile_Do_", 15, 15); -return x_1; -} -} -static lean_object* _init_l_Lean_doElemWhile__Do_____closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_unbracketedExplicitBinders___closed__1; -x_2 = l_Lean_doElemWhile__Do_____closed__1; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_doElemWhile__Do_____closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_unbracketedExplicitBinders___closed__5; -x_2 = l_Lean_doElemWhile___x3a__Do_____closed__4; -x_3 = l_Lean_doElemWhile___x3a__Do_____closed__9; -x_4 = lean_alloc_ctor(2, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; -} -} -static lean_object* _init_l_Lean_doElemWhile__Do_____closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_unbracketedExplicitBinders___closed__5; -x_2 = l_Lean_doElemWhile__Do_____closed__3; -x_3 = l_Lean_doElemWhile___x3a__Do_____closed__12; -x_4 = lean_alloc_ctor(2, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; -} -} -static lean_object* _init_l_Lean_doElemWhile__Do_____closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_unbracketedExplicitBinders___closed__5; -x_2 = l_Lean_doElemWhile__Do_____closed__4; -x_3 = l_Lean_doElemRepeat_____closed__7; -x_4 = lean_alloc_ctor(2, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; -} -} -static lean_object* _init_l_Lean_doElemWhile__Do_____closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_doElemWhile__Do_____closed__2; -x_2 = lean_unsigned_to_nat(1022u); -x_3 = l_Lean_doElemWhile__Do_____closed__5; -x_4 = lean_alloc_ctor(3, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; -} -} -static lean_object* _init_l_Lean_doElemWhile__Do__() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_doElemWhile__Do_____closed__6; -return x_1; -} -} -LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; uint8_t x_5; -x_4 = l_Lean_doElemWhile__Do_____closed__2; -lean_inc(x_1); -x_5 = l_Lean_Syntax_isOfKind(x_1, x_4); -if (x_5 == 0) -{ -lean_object* x_6; lean_object* x_7; -lean_dec(x_1); -x_6 = lean_box(1); -x_7 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_7, 0, x_6); -lean_ctor_set(x_7, 1, x_3); -return x_7; -} -else -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_8 = lean_unsigned_to_nat(1u); -x_9 = l_Lean_Syntax_getArg(x_1, x_8); -x_10 = lean_unsigned_to_nat(3u); -x_11 = l_Lean_Syntax_getArg(x_1, x_10); -lean_dec(x_1); -x_12 = lean_ctor_get(x_2, 5); -x_13 = 0; -x_14 = l_Lean_SourceInfo_fromRef(x_12, x_13); -x_15 = l___aux__Init__NotationExtra______macroRules__tacticFunext________1___closed__4; -lean_inc(x_14); -x_16 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_16, 0, x_14); -lean_ctor_set(x_16, 1, x_15); -x_17 = l_unexpandIte___closed__3; -lean_inc(x_14); -x_18 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_18, 0, x_14); -lean_ctor_set(x_18, 1, x_17); -x_19 = l_Lean_expandExplicitBindersAux_loop___closed__6; -x_20 = l_Lean_expandExplicitBindersAux_loop___closed__14; -lean_inc(x_14); -x_21 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_21, 0, x_14); -lean_ctor_set(x_21, 1, x_19); -lean_ctor_set(x_21, 2, x_20); -x_22 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8; -lean_inc(x_21); -lean_inc(x_14); -x_23 = l_Lean_Syntax_node2(x_14, x_22, x_21, x_9); -x_24 = l_unexpandIte___closed__4; -lean_inc(x_14); -x_25 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_25, 0, x_14); -lean_ctor_set(x_25, 1, x_24); -x_26 = l_unexpandIte___closed__5; -lean_inc(x_14); -x_27 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_27, 0, x_14); -lean_ctor_set(x_27, 1, x_26); -x_28 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11; -lean_inc(x_14); -x_29 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_29, 0, x_14); -lean_ctor_set(x_29, 1, x_28); -x_30 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10; -lean_inc(x_14); -x_31 = l_Lean_Syntax_node1(x_14, x_30, x_29); -x_32 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__4; -lean_inc(x_21); -lean_inc(x_14); -x_33 = l_Lean_Syntax_node2(x_14, x_32, x_31, x_21); -lean_inc(x_14); -x_34 = l_Lean_Syntax_node1(x_14, x_19, x_33); -x_35 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__2; -lean_inc(x_14); -x_36 = l_Lean_Syntax_node1(x_14, x_35, x_34); -lean_inc(x_14); -x_37 = l_Lean_Syntax_node2(x_14, x_19, x_27, x_36); -x_38 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__6; -lean_inc(x_21); -lean_inc(x_14); -x_39 = l_Lean_Syntax_node6(x_14, x_38, x_18, x_23, x_25, x_11, x_21, x_37); -lean_inc(x_14); -x_40 = l_Lean_Syntax_node2(x_14, x_32, x_39, x_21); -lean_inc(x_14); -x_41 = l_Lean_Syntax_node1(x_14, x_19, x_40); -lean_inc(x_14); -x_42 = l_Lean_Syntax_node1(x_14, x_35, x_41); -x_43 = l_Lean_doElemRepeat_____closed__2; -x_44 = l_Lean_Syntax_node2(x_14, x_43, x_16, x_42); -x_45 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_45, 0, x_44); -lean_ctor_set(x_45, 1, x_3); -return x_45; -} -} -} -LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1(x_1, x_2, x_3); -lean_dec(x_2); -return x_4; -} -} -static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("doElemRepeat__Until_", 20, 20); -return x_1; -} -} -static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_unbracketedExplicitBinders___closed__1; -x_2 = l_Lean_doElemRepeat____Until_____closed__1; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_unbracketedExplicitBinders___closed__5; -x_2 = l_Lean_doElemRepeat_____closed__8; -x_3 = l_Lean_solveTactic___closed__7; -x_4 = lean_alloc_ctor(2, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; -} -} -static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("until ", 6, 6); -return x_1; -} -} -static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_doElemRepeat____Until_____closed__4; -x_2 = lean_alloc_ctor(5, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_unbracketedExplicitBinders___closed__5; -x_2 = l_Lean_doElemRepeat____Until_____closed__3; -x_3 = l_Lean_doElemRepeat____Until_____closed__5; -x_4 = lean_alloc_ctor(2, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; -} -} -static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__7() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_unbracketedExplicitBinders___closed__5; -x_2 = l_Lean_doElemRepeat____Until_____closed__6; -x_3 = l_Lean_unbracketedExplicitBinders___closed__19; -x_4 = lean_alloc_ctor(2, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; -} -} -static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__8() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_doElemRepeat____Until_____closed__2; -x_2 = lean_unsigned_to_nat(1022u); -x_3 = l_Lean_doElemRepeat____Until_____closed__7; -x_4 = lean_alloc_ctor(3, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; -} -} -static lean_object* _init_l_Lean_doElemRepeat____Until__() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_doElemRepeat____Until_____closed__8; -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____Until____1___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("doNested", 8, 8); -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____Until____1___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_unbracketedExplicitBinders___closed__1; -x_2 = l_Lean_expandExplicitBindersAux_loop___closed__1; -x_3 = l_Lean_expandExplicitBindersAux_loop___closed__2; -x_4 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____Until____1___closed__1; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; -} -} -LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____Until____1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; uint8_t x_5; -x_4 = l_Lean_doElemRepeat____Until_____closed__2; -lean_inc(x_1); -x_5 = l_Lean_Syntax_isOfKind(x_1, x_4); -if (x_5 == 0) -{ -lean_object* x_6; lean_object* x_7; -lean_dec(x_1); -x_6 = lean_box(1); -x_7 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_7, 0, x_6); -lean_ctor_set(x_7, 1, x_3); -return x_7; -} -else -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_8 = lean_unsigned_to_nat(1u); -x_9 = l_Lean_Syntax_getArg(x_1, x_8); -x_10 = lean_unsigned_to_nat(3u); -x_11 = l_Lean_Syntax_getArg(x_1, x_10); -lean_dec(x_1); -x_12 = lean_ctor_get(x_2, 5); -x_13 = 0; -x_14 = l_Lean_SourceInfo_fromRef(x_12, x_13); -x_15 = l___aux__Init__NotationExtra______macroRules__tacticFunext________1___closed__4; -lean_inc(x_14); -x_16 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_16, 0, x_14); -lean_ctor_set(x_16, 1, x_15); -x_17 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__17; -lean_inc(x_14); -x_18 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_18, 0, x_14); -lean_ctor_set(x_18, 1, x_17); -x_19 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____Until____1___closed__2; -lean_inc(x_14); -x_20 = l_Lean_Syntax_node2(x_14, x_19, x_18, x_9); -x_21 = l___aux__Init__NotationExtra______macroRules__tacticFunext________1___lambda__2___closed__9; -lean_inc(x_14); -x_22 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_22, 0, x_14); -lean_ctor_set(x_22, 1, x_21); -x_23 = l_Lean_expandExplicitBindersAux_loop___closed__6; -lean_inc(x_14); -x_24 = l_Lean_Syntax_node1(x_14, x_23, x_22); -x_25 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__4; -lean_inc(x_14); -x_26 = l_Lean_Syntax_node2(x_14, x_25, x_20, x_24); -x_27 = l_unexpandIte___closed__3; -lean_inc(x_14); -x_28 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_28, 0, x_14); -lean_ctor_set(x_28, 1, x_27); -x_29 = l_Lean_expandExplicitBindersAux_loop___closed__14; -lean_inc(x_14); -x_30 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_30, 0, x_14); -lean_ctor_set(x_30, 1, x_23); -lean_ctor_set(x_30, 2, x_29); -x_31 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8; -lean_inc(x_30); -lean_inc(x_14); -x_32 = l_Lean_Syntax_node2(x_14, x_31, x_30, x_11); -x_33 = l_unexpandIte___closed__4; -lean_inc(x_14); -x_34 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_34, 0, x_14); -lean_ctor_set(x_34, 1, x_33); -x_35 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11; -lean_inc(x_14); -x_36 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_36, 0, x_14); -lean_ctor_set(x_36, 1, x_35); -x_37 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10; -lean_inc(x_14); -x_38 = l_Lean_Syntax_node1(x_14, x_37, x_36); -lean_inc(x_30); -lean_inc(x_14); -x_39 = l_Lean_Syntax_node2(x_14, x_25, x_38, x_30); -lean_inc(x_14); -x_40 = l_Lean_Syntax_node1(x_14, x_23, x_39); -x_41 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__2; -lean_inc(x_14); -x_42 = l_Lean_Syntax_node1(x_14, x_41, x_40); -x_43 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__6; -lean_inc_n(x_30, 2); -lean_inc(x_14); -x_44 = l_Lean_Syntax_node6(x_14, x_43, x_28, x_32, x_34, x_42, x_30, x_30); -lean_inc(x_14); -x_45 = l_Lean_Syntax_node2(x_14, x_25, x_44, x_30); -lean_inc(x_14); -x_46 = l_Lean_Syntax_node2(x_14, x_23, x_26, x_45); -lean_inc(x_14); -x_47 = l_Lean_Syntax_node1(x_14, x_41, x_46); -x_48 = l_Lean_doElemRepeat_____closed__2; -x_49 = l_Lean_Syntax_node2(x_14, x_48, x_16, x_47); -x_50 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_50, 0, x_49); -lean_ctor_set(x_50, 1, x_3); -return x_50; -} -} -} -LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____Until____1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____Until____1(x_1, x_2, x_3); -lean_dec(x_2); -return x_4; -} -} -static lean_object* _init_l_Lean_term__Matches___x7c___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("term_Matches_|", 14, 14); -return x_1; -} -} -static lean_object* _init_l_Lean_term__Matches___x7c___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_unbracketedExplicitBinders___closed__1; -x_2 = l_Lean_term__Matches___x7c___closed__1; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_term__Matches___x7c___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked(" matches ", 9, 9); -return x_1; -} -} -static lean_object* _init_l_Lean_term__Matches___x7c___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_term__Matches___x7c___closed__3; -x_2 = lean_alloc_ctor(5, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_term__Matches___x7c___closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_unbracketedExplicitBinders___closed__18; -x_2 = lean_unsigned_to_nat(51u); -x_3 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_term__Matches___x7c___closed__6() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked(" | ", 3, 3); -return x_1; -} -} -static lean_object* _init_l_Lean_term__Matches___x7c___closed__7() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_term__Matches___x7c___closed__6; -x_2 = lean_alloc_ctor(5, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_term__Matches___x7c___closed__8() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; -x_1 = l_Lean_term__Matches___x7c___closed__5; -x_2 = l_Lean_term__Matches___x7c___closed__6; -x_3 = l_Lean_term__Matches___x7c___closed__7; -x_4 = 0; -x_5 = lean_alloc_ctor(11, 3, 1); -lean_ctor_set(x_5, 0, x_1); -lean_ctor_set(x_5, 1, x_2); -lean_ctor_set(x_5, 2, x_3); -lean_ctor_set_uint8(x_5, sizeof(void*)*3, x_4); -return x_5; -} -} -static lean_object* _init_l_Lean_term__Matches___x7c___closed__9() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_unbracketedExplicitBinders___closed__5; -x_2 = l_Lean_term__Matches___x7c___closed__4; -x_3 = l_Lean_term__Matches___x7c___closed__8; -x_4 = lean_alloc_ctor(2, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; -} -} -static lean_object* _init_l_Lean_term__Matches___x7c___closed__10() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_term__Matches___x7c___closed__2; -x_2 = lean_unsigned_to_nat(50u); -x_3 = lean_unsigned_to_nat(51u); -x_4 = l_Lean_term__Matches___x7c___closed__9; -x_5 = lean_alloc_ctor(4, 4, 0); -lean_ctor_set(x_5, 0, x_1); -lean_ctor_set(x_5, 1, x_2); -lean_ctor_set(x_5, 2, x_3); -lean_ctor_set(x_5, 3, x_4); -return x_5; -} -} -static lean_object* _init_l_Lean_term__Matches___x7c() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_term__Matches___x7c___closed__10; -return x_1; -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___spec__1(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { -_start: -{ -uint8_t x_6; -x_6 = lean_usize_dec_lt(x_4, x_3); -if (x_6 == 0) -{ -lean_dec(x_2); -lean_dec(x_1); -return x_5; -} -else -{ -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; size_t x_11; size_t x_12; lean_object* x_13; -x_7 = lean_array_uget(x_5, x_4); -x_8 = lean_unsigned_to_nat(0u); -x_9 = lean_array_uset(x_5, x_4, x_8); -lean_inc(x_2); -lean_inc(x_1); -x_10 = l_Lean_Syntax_node1(x_1, x_2, x_7); -x_11 = 1; -x_12 = lean_usize_add(x_4, x_11); -x_13 = lean_array_uset(x_9, x_4, x_10); -x_4 = x_12; -x_5 = x_13; -goto _start; -} -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_unbracketedExplicitBinders___closed__1; -x_2 = l_Lean_expandExplicitBindersAux_loop___closed__1; -x_3 = l_Lean_expandExplicitBindersAux_loop___closed__2; -x_4 = l___aux__Init__NotationExtra______macroRules__tacticFunext________1___closed__5; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__2() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("match", 5, 5); -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_unbracketedExplicitBinders___closed__1; -x_2 = l_Lean_expandExplicitBindersAux_loop___closed__1; -x_3 = l_Lean_expandExplicitBindersAux_loop___closed__2; -x_4 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__2; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("matchDiscr", 10, 10); -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_unbracketedExplicitBinders___closed__1; -x_2 = l_Lean_expandExplicitBindersAux_loop___closed__1; -x_3 = l_Lean_expandExplicitBindersAux_loop___closed__2; -x_4 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__4; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__6() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("with", 4, 4); -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__7() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("matchAlts", 9, 9); -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__8() { +static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; @@ -18036,6 +16557,7 @@ lean_object* initialize_Init_Data_ToString_Basic(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_Array_Subarray(uint8_t builtin, lean_object*); lean_object* initialize_Init_Conv(uint8_t builtin, lean_object*); lean_object* initialize_Init_Meta(uint8_t builtin, lean_object*); +lean_object* initialize_Init_While(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Init_NotationExtra(uint8_t builtin, lean_object* w) { lean_object * res; @@ -18053,6 +16575,9 @@ lean_dec_ref(res); res = initialize_Init_Meta(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +res = initialize_Init_While(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_unbracketedExplicitBinders___closed__1 = _init_l_Lean_unbracketedExplicitBinders___closed__1(); lean_mark_persistent(l_Lean_unbracketedExplicitBinders___closed__1); l_Lean_unbracketedExplicitBinders___closed__2 = _init_l_Lean_unbracketedExplicitBinders___closed__2(); @@ -19147,150 +17672,6 @@ l_Lean___aux__Init__NotationExtra______macroRules__Lean__solveTactic__1___closed lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__solveTactic__1___closed__4); l_Lean___aux__Init__NotationExtra______macroRules__Lean__solveTactic__1___closed__5 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__solveTactic__1___closed__5(); lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__solveTactic__1___closed__5); -l_Lean_doElemRepeat_____closed__1 = _init_l_Lean_doElemRepeat_____closed__1(); -lean_mark_persistent(l_Lean_doElemRepeat_____closed__1); -l_Lean_doElemRepeat_____closed__2 = _init_l_Lean_doElemRepeat_____closed__2(); -lean_mark_persistent(l_Lean_doElemRepeat_____closed__2); -l_Lean_doElemRepeat_____closed__3 = _init_l_Lean_doElemRepeat_____closed__3(); -lean_mark_persistent(l_Lean_doElemRepeat_____closed__3); -l_Lean_doElemRepeat_____closed__4 = _init_l_Lean_doElemRepeat_____closed__4(); -lean_mark_persistent(l_Lean_doElemRepeat_____closed__4); -l_Lean_doElemRepeat_____closed__5 = _init_l_Lean_doElemRepeat_____closed__5(); -lean_mark_persistent(l_Lean_doElemRepeat_____closed__5); -l_Lean_doElemRepeat_____closed__6 = _init_l_Lean_doElemRepeat_____closed__6(); -lean_mark_persistent(l_Lean_doElemRepeat_____closed__6); -l_Lean_doElemRepeat_____closed__7 = _init_l_Lean_doElemRepeat_____closed__7(); -lean_mark_persistent(l_Lean_doElemRepeat_____closed__7); -l_Lean_doElemRepeat_____closed__8 = _init_l_Lean_doElemRepeat_____closed__8(); -lean_mark_persistent(l_Lean_doElemRepeat_____closed__8); -l_Lean_doElemRepeat_____closed__9 = _init_l_Lean_doElemRepeat_____closed__9(); -lean_mark_persistent(l_Lean_doElemRepeat_____closed__9); -l_Lean_doElemRepeat__ = _init_l_Lean_doElemRepeat__(); -lean_mark_persistent(l_Lean_doElemRepeat__); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__1 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__1(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__1); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__2 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__2(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__2); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__3 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__3(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__3); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__4 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__4(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__4); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__5 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__5(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__5); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__6 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__6(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__6); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__7 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__7(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__7); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__8 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__8(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__8); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__9 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__9(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__9); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__10 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__10(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__10); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__11 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__11(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__11); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__12 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__12(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__12); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__13 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__13(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__13); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__14 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__14(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__14); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__15 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__15(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__15); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__16 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__16(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__16); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__17 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__17(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__17); -l_Lean_doElemWhile___x3a__Do_____closed__1 = _init_l_Lean_doElemWhile___x3a__Do_____closed__1(); -lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__1); -l_Lean_doElemWhile___x3a__Do_____closed__2 = _init_l_Lean_doElemWhile___x3a__Do_____closed__2(); -lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__2); -l_Lean_doElemWhile___x3a__Do_____closed__3 = _init_l_Lean_doElemWhile___x3a__Do_____closed__3(); -lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__3); -l_Lean_doElemWhile___x3a__Do_____closed__4 = _init_l_Lean_doElemWhile___x3a__Do_____closed__4(); -lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__4); -l_Lean_doElemWhile___x3a__Do_____closed__5 = _init_l_Lean_doElemWhile___x3a__Do_____closed__5(); -lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__5); -l_Lean_doElemWhile___x3a__Do_____closed__6 = _init_l_Lean_doElemWhile___x3a__Do_____closed__6(); -lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__6); -l_Lean_doElemWhile___x3a__Do_____closed__7 = _init_l_Lean_doElemWhile___x3a__Do_____closed__7(); -lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__7); -l_Lean_doElemWhile___x3a__Do_____closed__8 = _init_l_Lean_doElemWhile___x3a__Do_____closed__8(); -lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__8); -l_Lean_doElemWhile___x3a__Do_____closed__9 = _init_l_Lean_doElemWhile___x3a__Do_____closed__9(); -lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__9); -l_Lean_doElemWhile___x3a__Do_____closed__10 = _init_l_Lean_doElemWhile___x3a__Do_____closed__10(); -lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__10); -l_Lean_doElemWhile___x3a__Do_____closed__11 = _init_l_Lean_doElemWhile___x3a__Do_____closed__11(); -lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__11); -l_Lean_doElemWhile___x3a__Do_____closed__12 = _init_l_Lean_doElemWhile___x3a__Do_____closed__12(); -lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__12); -l_Lean_doElemWhile___x3a__Do_____closed__13 = _init_l_Lean_doElemWhile___x3a__Do_____closed__13(); -lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__13); -l_Lean_doElemWhile___x3a__Do_____closed__14 = _init_l_Lean_doElemWhile___x3a__Do_____closed__14(); -lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__14); -l_Lean_doElemWhile___x3a__Do_____closed__15 = _init_l_Lean_doElemWhile___x3a__Do_____closed__15(); -lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__15); -l_Lean_doElemWhile___x3a__Do__ = _init_l_Lean_doElemWhile___x3a__Do__(); -lean_mark_persistent(l_Lean_doElemWhile___x3a__Do__); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__2 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__2(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__2); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__4 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__4(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__4); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__6 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__6(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__6); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__9 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__9(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__9); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11); -l_Lean_doElemWhile__Do_____closed__1 = _init_l_Lean_doElemWhile__Do_____closed__1(); -lean_mark_persistent(l_Lean_doElemWhile__Do_____closed__1); -l_Lean_doElemWhile__Do_____closed__2 = _init_l_Lean_doElemWhile__Do_____closed__2(); -lean_mark_persistent(l_Lean_doElemWhile__Do_____closed__2); -l_Lean_doElemWhile__Do_____closed__3 = _init_l_Lean_doElemWhile__Do_____closed__3(); -lean_mark_persistent(l_Lean_doElemWhile__Do_____closed__3); -l_Lean_doElemWhile__Do_____closed__4 = _init_l_Lean_doElemWhile__Do_____closed__4(); -lean_mark_persistent(l_Lean_doElemWhile__Do_____closed__4); -l_Lean_doElemWhile__Do_____closed__5 = _init_l_Lean_doElemWhile__Do_____closed__5(); -lean_mark_persistent(l_Lean_doElemWhile__Do_____closed__5); -l_Lean_doElemWhile__Do_____closed__6 = _init_l_Lean_doElemWhile__Do_____closed__6(); -lean_mark_persistent(l_Lean_doElemWhile__Do_____closed__6); -l_Lean_doElemWhile__Do__ = _init_l_Lean_doElemWhile__Do__(); -lean_mark_persistent(l_Lean_doElemWhile__Do__); -l_Lean_doElemRepeat____Until_____closed__1 = _init_l_Lean_doElemRepeat____Until_____closed__1(); -lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__1); -l_Lean_doElemRepeat____Until_____closed__2 = _init_l_Lean_doElemRepeat____Until_____closed__2(); -lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__2); -l_Lean_doElemRepeat____Until_____closed__3 = _init_l_Lean_doElemRepeat____Until_____closed__3(); -lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__3); -l_Lean_doElemRepeat____Until_____closed__4 = _init_l_Lean_doElemRepeat____Until_____closed__4(); -lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__4); -l_Lean_doElemRepeat____Until_____closed__5 = _init_l_Lean_doElemRepeat____Until_____closed__5(); -lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__5); -l_Lean_doElemRepeat____Until_____closed__6 = _init_l_Lean_doElemRepeat____Until_____closed__6(); -lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__6); -l_Lean_doElemRepeat____Until_____closed__7 = _init_l_Lean_doElemRepeat____Until_____closed__7(); -lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__7); -l_Lean_doElemRepeat____Until_____closed__8 = _init_l_Lean_doElemRepeat____Until_____closed__8(); -lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__8); -l_Lean_doElemRepeat____Until__ = _init_l_Lean_doElemRepeat____Until__(); -lean_mark_persistent(l_Lean_doElemRepeat____Until__); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____Until____1___closed__1 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____Until____1___closed__1(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____Until____1___closed__1); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____Until____1___closed__2 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____Until____1___closed__2(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____Until____1___closed__2); l_Lean_term__Matches___x7c___closed__1 = _init_l_Lean_term__Matches___x7c___closed__1(); lean_mark_persistent(l_Lean_term__Matches___x7c___closed__1); l_Lean_term__Matches___x7c___closed__2 = _init_l_Lean_term__Matches___x7c___closed__2(); diff --git a/stage0/stdlib/Init/System/FilePath.c b/stage0/stdlib/Init/System/FilePath.c index 9c0fe203490f..383cb73cd5a9 100644 --- a/stage0/stdlib/Init/System/FilePath.c +++ b/stage0/stdlib/Init/System/FilePath.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Init.System.FilePath -// Imports: Init.System.Platform Init.Data.String.Basic Init.Data.Repr Init.Data.ToString.Basic +// Imports: Init.System.Platform Init.Data.ToString.Basic #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -1976,8 +1976,6 @@ return x_5; } } lean_object* initialize_Init_System_Platform(uint8_t builtin, lean_object*); -lean_object* initialize_Init_Data_String_Basic(uint8_t builtin, lean_object*); -lean_object* initialize_Init_Data_Repr(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_ToString_Basic(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Init_System_FilePath(uint8_t builtin, lean_object* w) { @@ -1987,12 +1985,6 @@ _G_initialized = true; res = initialize_Init_System_Platform(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -res = initialize_Init_Data_String_Basic(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -res = initialize_Init_Data_Repr(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Init_Data_ToString_Basic(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Init/System/IO.c b/stage0/stdlib/Init/System/IO.c index 48f281ef6fed..4aab07c4f0ab 100644 --- a/stage0/stdlib/Init/System/IO.c +++ b/stage0/stdlib/Init/System/IO.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Init.System.IO -// Imports: Init.Control.Reader Init.Data.String Init.Data.ByteArray Init.System.IOError Init.System.FilePath Init.System.ST Init.Data.ToString.Macro Init.Data.Ord +// Imports: Init.System.IOError Init.System.FilePath Init.System.ST Init.Data.Ord #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -11497,28 +11497,15 @@ return x_89; } } } -lean_object* initialize_Init_Control_Reader(uint8_t builtin, lean_object*); -lean_object* initialize_Init_Data_String(uint8_t builtin, lean_object*); -lean_object* initialize_Init_Data_ByteArray(uint8_t builtin, lean_object*); lean_object* initialize_Init_System_IOError(uint8_t builtin, lean_object*); lean_object* initialize_Init_System_FilePath(uint8_t builtin, lean_object*); lean_object* initialize_Init_System_ST(uint8_t builtin, lean_object*); -lean_object* initialize_Init_Data_ToString_Macro(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_Ord(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Init_System_IO(uint8_t builtin, lean_object* w) { lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init_Control_Reader(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -res = initialize_Init_Data_String(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -res = initialize_Init_Data_ByteArray(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Init_System_IOError(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); @@ -11528,9 +11515,6 @@ lean_dec_ref(res); res = initialize_Init_System_ST(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -res = initialize_Init_Data_ToString_Macro(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Init_Data_Ord(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Init/System/IOError.c b/stage0/stdlib/Init/System/IOError.c index 798856d2ab29..aea8986c7cbf 100644 --- a/stage0/stdlib/Init/System/IOError.c +++ b/stage0/stdlib/Init/System/IOError.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Init.System.IOError -// Imports: Init.Core Init.Data.UInt.Basic Init.Data.ToString.Basic Init.Data.String.Basic +// Imports: Init.Data.ToString.Basic #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -1420,27 +1420,15 @@ x_1 = l_IO_Error_instToString___closed__1; return x_1; } } -lean_object* initialize_Init_Core(uint8_t builtin, lean_object*); -lean_object* initialize_Init_Data_UInt_Basic(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_ToString_Basic(uint8_t builtin, lean_object*); -lean_object* initialize_Init_Data_String_Basic(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Init_System_IOError(uint8_t builtin, lean_object* w) { lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init_Core(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -res = initialize_Init_Data_UInt_Basic(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Init_Data_ToString_Basic(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -res = initialize_Init_Data_String_Basic(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); l_IO_instInhabitedError___closed__1 = _init_l_IO_instInhabitedError___closed__1(); l_IO_instInhabitedError___closed__2 = _init_l_IO_instInhabitedError___closed__2(); lean_mark_persistent(l_IO_instInhabitedError___closed__2); diff --git a/stage0/stdlib/Init/Tactics.c b/stage0/stdlib/Init/Tactics.c index cefc8c1aee82..7ddcdaab450e 100644 --- a/stage0/stdlib/Init/Tactics.c +++ b/stage0/stdlib/Init/Tactics.c @@ -4257,64 +4257,67 @@ return x_7; } else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_8 = lean_unsigned_to_nat(1u); +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; uint8_t x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_8 = lean_unsigned_to_nat(0u); x_9 = l_Lean_Syntax_getArg(x_1, x_8); -x_10 = lean_unsigned_to_nat(2u); +x_10 = lean_unsigned_to_nat(1u); x_11 = l_Lean_Syntax_getArg(x_1, x_10); -x_12 = lean_unsigned_to_nat(3u); +x_12 = lean_unsigned_to_nat(2u); x_13 = l_Lean_Syntax_getArg(x_1, x_12); +x_14 = lean_unsigned_to_nat(3u); +x_15 = l_Lean_Syntax_getArg(x_1, x_14); lean_dec(x_1); -x_14 = l_Lean_Syntax_getArgs(x_9); +x_16 = l_Lean_Syntax_getArgs(x_11); +lean_dec(x_11); +x_17 = lean_ctor_get(x_2, 5); +x_18 = l_Lean_replaceRef(x_13, x_17); +x_19 = 0; +x_20 = l_Lean_SourceInfo_fromRef(x_18, x_19); +lean_dec(x_18); +x_21 = 1; +x_22 = l_Lean_SourceInfo_fromRef(x_9, x_21); lean_dec(x_9); -x_15 = lean_ctor_get(x_2, 5); -x_16 = l_Lean_replaceRef(x_11, x_15); -x_17 = 0; -x_18 = l_Lean_SourceInfo_fromRef(x_16, x_17); +x_23 = l_Lean_Parser_Tactic_case___closed__1; +x_24 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); +x_25 = l_Lean_Parser_Tactic___aux__Init__Tactics______macroRules__Lean__Parser__Tactic__tacticExfalso__1___closed__16; +lean_inc(x_20); +x_26 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_26, 0, x_20); +lean_ctor_set(x_26, 1, x_25); +x_27 = l_Lean_Parser_Tactic___aux__Init__Tactics______macroRules__Lean__Parser__Tactic__tacticNext___x3d_x3e____1___closed__5; +lean_inc(x_20); +x_28 = l_Lean_Syntax_node1(x_20, x_27, x_26); +x_29 = l_Lean_Parser_Tactic___aux__Init__Tactics______macroRules__Lean__Parser__Tactic__tacticNext___x3d_x3e____1___closed__2; +lean_inc(x_20); +x_30 = l_Lean_Syntax_node1(x_20, x_29, x_28); +x_31 = l_Lean_Parser_Tactic___aux__Init__Tactics______macroRules__Lean__Parser__Tactic__tacticNext___x3d_x3e____1___closed__6; +x_32 = l_Array_appendCore___rarg(x_31, x_16); lean_dec(x_16); -x_19 = l_Lean_Parser_Tactic_case___closed__1; -lean_inc(x_18); -x_20 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_20, 0, x_18); -lean_ctor_set(x_20, 1, x_19); -x_21 = l_Lean_Parser_Tactic___aux__Init__Tactics______macroRules__Lean__Parser__Tactic__tacticExfalso__1___closed__16; -lean_inc(x_18); -x_22 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_22, 0, x_18); -lean_ctor_set(x_22, 1, x_21); -x_23 = l_Lean_Parser_Tactic___aux__Init__Tactics______macroRules__Lean__Parser__Tactic__tacticNext___x3d_x3e____1___closed__5; -lean_inc(x_18); -x_24 = l_Lean_Syntax_node1(x_18, x_23, x_22); -x_25 = l_Lean_Parser_Tactic___aux__Init__Tactics______macroRules__Lean__Parser__Tactic__tacticNext___x3d_x3e____1___closed__2; -lean_inc(x_18); -x_26 = l_Lean_Syntax_node1(x_18, x_25, x_24); -x_27 = l_Lean_Parser_Tactic___aux__Init__Tactics______macroRules__Lean__Parser__Tactic__tacticNext___x3d_x3e____1___closed__6; -x_28 = l_Array_appendCore___rarg(x_27, x_14); -lean_dec(x_14); -x_29 = l_Lean_Parser_Tactic___aux__Init__Tactics______macroRules__Lean__Parser__Tactic__tacticExfalso__1___closed__12; -lean_inc(x_18); -x_30 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_30, 0, x_18); -lean_ctor_set(x_30, 1, x_29); -lean_ctor_set(x_30, 2, x_28); -x_31 = l_Lean_Parser_Tactic___aux__Init__Tactics______macroRules__Lean__Parser__Tactic__tacticNext___x3d_x3e____1___closed__4; -lean_inc(x_18); -x_32 = l_Lean_Syntax_node2(x_18, x_31, x_26, x_30); -lean_inc(x_18); -x_33 = l_Lean_Syntax_node1(x_18, x_29, x_32); -x_34 = 1; -x_35 = l_Lean_SourceInfo_fromRef(x_11, x_34); -lean_dec(x_11); -x_36 = l_Lean_Parser_Tactic___aux__Init__Tactics______macroRules__Lean__Parser__Tactic__tacticNext___x3d_x3e____1___closed__7; -x_37 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -x_38 = l_Lean_Parser_Tactic_case___closed__2; -x_39 = l_Lean_Syntax_node4(x_18, x_38, x_20, x_33, x_37, x_13); -x_40 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_40, 0, x_39); -lean_ctor_set(x_40, 1, x_3); -return x_40; +x_33 = l_Lean_Parser_Tactic___aux__Init__Tactics______macroRules__Lean__Parser__Tactic__tacticExfalso__1___closed__12; +lean_inc(x_20); +x_34 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_34, 0, x_20); +lean_ctor_set(x_34, 1, x_33); +lean_ctor_set(x_34, 2, x_32); +x_35 = l_Lean_Parser_Tactic___aux__Init__Tactics______macroRules__Lean__Parser__Tactic__tacticNext___x3d_x3e____1___closed__4; +lean_inc(x_20); +x_36 = l_Lean_Syntax_node2(x_20, x_35, x_30, x_34); +lean_inc(x_20); +x_37 = l_Lean_Syntax_node1(x_20, x_33, x_36); +x_38 = l_Lean_SourceInfo_fromRef(x_13, x_21); +lean_dec(x_13); +x_39 = l_Lean_Parser_Tactic___aux__Init__Tactics______macroRules__Lean__Parser__Tactic__tacticNext___x3d_x3e____1___closed__7; +x_40 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +x_41 = l_Lean_Parser_Tactic_case___closed__2; +x_42 = l_Lean_Syntax_node4(x_20, x_41, x_24, x_37, x_40, x_15); +x_43 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_43, 0, x_42); +lean_ctor_set(x_43, 1, x_3); +return x_43; } } } diff --git a/stage0/stdlib/Init/While.c b/stage0/stdlib/Init/While.c new file mode 100644 index 000000000000..cbdb412116c6 --- /dev/null +++ b/stage0/stdlib/Init/While.c @@ -0,0 +1,1980 @@ +// Lean compiler output +// Module: Init.While +// Imports: Init.Core +#include +#if defined(__clang__) +#pragma clang diagnostic ignored "-Wunused-parameter" +#pragma clang diagnostic ignored "-Wunused-label" +#elif defined(__GNUC__) && !defined(__CLANG__) +#pragma GCC diagnostic ignored "-Wunused-parameter" +#pragma GCC diagnostic ignored "-Wunused-label" +#pragma GCC diagnostic ignored "-Wunused-but-set-variable" +#endif +#ifdef __cplusplus +extern "C" { +#endif +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__3; +static lean_object* l_Lean_doElemRepeat____Until_____closed__10; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__10; +LEAN_EXPORT lean_object* l_Lean_Loop_toCtorIdx___boxed(lean_object*); +lean_object* lean_mk_empty_array_with_capacity(lean_object*); +static lean_object* l_Lean_doElemRepeat_____closed__11; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__8; +static lean_object* l_Lean_doElemRepeat____Until_____closed__11; +static lean_object* l_Lean_doElemRepeat_____closed__12; +static lean_object* l_Lean_doElemRepeat____Until_____closed__8; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__3; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__1; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__4; +LEAN_EXPORT lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_doElemRepeat____Until_____closed__12; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8; +LEAN_EXPORT lean_object* l_Lean_Loop_forIn___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_doElemRepeat_____closed__1; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11; +static lean_object* l_Lean_doElemRepeat____Until_____closed__5; +uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_instForInLoopUnit___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__2; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__11; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__23; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__14; +LEAN_EXPORT lean_object* l_Lean_instForInLoopUnit(lean_object*, lean_object*); +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__13; +LEAN_EXPORT lean_object* l_Lean_doElemRepeat____Until__; +static lean_object* l_Lean_doElemRepeat____Until_____closed__9; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__6; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__14; +lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_doElemRepeat_____closed__8; +static lean_object* l_Lean_doElemRepeat_____closed__2; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__18; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__11; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__9; +LEAN_EXPORT lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile__Do____1___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__18; +lean_object* l_Lean_SourceInfo_fromRef(lean_object*, uint8_t); +lean_object* l_Lean_Syntax_node6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_doElemRepeat_____closed__10; +LEAN_EXPORT lean_object* l_Lean_Loop_noConfusion___rarg(lean_object*); +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__13; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__25; +static lean_object* l_Lean_doElemRepeat____Until_____closed__15; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__8; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__17; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__22; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7; +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___rarg___lambda__1(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_doElemRepeat____Until_____closed__4; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5; +static lean_object* l_Lean_doElemRepeat____Until_____closed__17; +static lean_object* l_Lean_doElemWhile__Do_____closed__2; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__17; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__2; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__6; +static lean_object* l_Lean_doElemRepeat____Until_____closed__6; +lean_object* l_Lean_addMacroScope(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__16; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__19; +lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); +static lean_object* l_Lean_doElemWhile__Do_____closed__1; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__2; +lean_object* l_Lean_Syntax_node2(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___closed__2; +lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); +static lean_object* l_Lean_doElemRepeat____Until_____closed__16; +LEAN_EXPORT lean_object* l_Lean_Loop_noConfusion___rarg___boxed(lean_object*); +static lean_object* l_Lean_doElemRepeat_____closed__6; +LEAN_EXPORT lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile__Do____1(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__9; +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Loop_noConfusion(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_doElemRepeat____Until_____closed__7; +lean_object* l_Lean_Syntax_node4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_doElemRepeat_____closed__5; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__7; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1; +static lean_object* l_Lean_doElemRepeat____Until_____closed__3; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__19; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__4; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__12; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__21; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__6; +static lean_object* l_Lean_doElemRepeat____Until_____closed__2; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__15; +lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__4; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__20; +lean_object* l_Lean_Syntax_node1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_instForInLoopUnit___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_doElemWhile__Do_____closed__3; +static lean_object* l_Lean_doElemWhile__Do_____closed__6; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__12; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__16; +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___rarg(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__12; +static lean_object* l_Lean_doElemWhile__Do_____closed__5; +static lean_object* l_Lean_doElemRepeat_____closed__7; +LEAN_EXPORT lean_object* l_Lean_Loop_toCtorIdx(lean_object*); +LEAN_EXPORT lean_object* l_Lean_doElemRepeat__; +LEAN_EXPORT lean_object* l_Lean_Loop_forIn___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_doElemRepeat_____closed__3; +LEAN_EXPORT lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_doElemRepeat____Until_____closed__1; +LEAN_EXPORT lean_object* l_Lean_doElemWhile___x3a__Do__; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__15; +LEAN_EXPORT lean_object* l_Lean_Loop_noConfusion___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___closed__3; +LEAN_EXPORT lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__10; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__16; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___closed__1; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__5; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__5; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__20; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__13; +LEAN_EXPORT lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1(lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_doElemRepeat____Until_____closed__13; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__1; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__9; +LEAN_EXPORT lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_doElemWhile__Do__; +static lean_object* l_Lean_doElemRepeat_____closed__4; +static lean_object* l_Lean_doElemRepeat_____closed__9; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__7; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__24; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__15; +lean_object* l_String_toSubstring_x27(lean_object*); +static lean_object* l_Lean_doElemWhile__Do_____closed__4; +static lean_object* l_Lean_doElemRepeat____Until_____closed__14; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__14; +LEAN_EXPORT lean_object* l_Lean_Loop_forIn(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Loop_toCtorIdx(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_unsigned_to_nat(0u); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Loop_toCtorIdx___boxed(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = l_Lean_Loop_toCtorIdx(x_1); +lean_dec(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Loop_noConfusion___rarg(lean_object* x_1) { +_start: +{ +lean_inc(x_1); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Loop_noConfusion(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = lean_alloc_closure((void*)(l_Lean_Loop_noConfusion___rarg___boxed), 1, 0); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_Loop_noConfusion___rarg___boxed(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = l_Lean_Loop_noConfusion___rarg(x_1); +lean_dec(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Loop_noConfusion___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Lean_Loop_noConfusion(x_1, x_2, x_3, x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +if (lean_obj_tag(x_3) == 0) +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +lean_dec(x_2); +x_4 = lean_ctor_get(x_3, 0); +lean_inc(x_4); +lean_dec(x_3); +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_apply_2(x_6, lean_box(0), x_4); +return x_7; +} +else +{ +lean_object* x_8; lean_object* x_9; +x_8 = lean_ctor_get(x_3, 0); +lean_inc(x_8); +lean_dec(x_3); +x_9 = l_Lean_Loop_forIn_loop___rarg(x_1, x_2, x_8); +return x_9; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_4 = lean_ctor_get(x_1, 1); +lean_inc(x_4); +x_5 = lean_box(0); +lean_inc(x_2); +x_6 = lean_apply_2(x_2, x_5, x_3); +x_7 = lean_alloc_closure((void*)(l_Lean_Loop_forIn_loop___rarg___lambda__1), 3, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +x_8 = lean_apply_4(x_4, lean_box(0), lean_box(0), x_6, x_7); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Lean_Loop_forIn_loop___rarg), 3, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Loop_forIn___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Lean_Loop_forIn_loop___rarg(x_1, x_4, x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_Loop_forIn(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Lean_Loop_forIn___rarg___boxed), 4, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Loop_forIn___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Lean_Loop_forIn___rarg(x_1, x_2, x_3, x_4); +lean_dec(x_2); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_instForInLoopUnit___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Lean_Loop_forIn_loop___rarg(x_1, x_4, x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_instForInLoopUnit(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Lean_instForInLoopUnit___rarg___boxed), 4, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_instForInLoopUnit___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Lean_instForInLoopUnit___rarg(x_1, x_2, x_3, x_4); +lean_dec(x_2); +return x_5; +} +} +static lean_object* _init_l_Lean_doElemRepeat_____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_doElemRepeat_____closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("doElemRepeat_", 13, 13); +return x_1; +} +} +static lean_object* _init_l_Lean_doElemRepeat_____closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_doElemRepeat_____closed__1; +x_2 = l_Lean_doElemRepeat_____closed__2; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_doElemRepeat_____closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("andthen", 7, 7); +return x_1; +} +} +static lean_object* _init_l_Lean_doElemRepeat_____closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_doElemRepeat_____closed__4; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_doElemRepeat_____closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("repeat ", 7, 7); +return x_1; +} +} +static lean_object* _init_l_Lean_doElemRepeat_____closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_doElemRepeat_____closed__6; +x_2 = lean_alloc_ctor(5, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_doElemRepeat_____closed__8() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("doSeq", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean_doElemRepeat_____closed__9() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_doElemRepeat_____closed__8; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_doElemRepeat_____closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_doElemRepeat_____closed__9; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_doElemRepeat_____closed__11() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemRepeat_____closed__5; +x_2 = l_Lean_doElemRepeat_____closed__7; +x_3 = l_Lean_doElemRepeat_____closed__10; +x_4 = lean_alloc_ctor(2, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_doElemRepeat_____closed__12() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemRepeat_____closed__3; +x_2 = lean_unsigned_to_nat(1022u); +x_3 = l_Lean_doElemRepeat_____closed__11; +x_4 = lean_alloc_ctor(3, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_doElemRepeat__() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_doElemRepeat_____closed__12; +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Parser", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Term", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("doFor", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_doElemRepeat_____closed__1; +x_2 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__1; +x_3 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__2; +x_4 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__3; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("for", 3, 3); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("null", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__6; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__8() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("doForDecl", 9, 9); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__9() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_doElemRepeat_____closed__1; +x_2 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__1; +x_3 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__2; +x_4 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__8; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(0u); +x_2 = lean_mk_empty_array_with_capacity(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__11() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("hole", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__12() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_doElemRepeat_____closed__1; +x_2 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__1; +x_3 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__2; +x_4 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__11; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__13() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("_", 1, 1); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__14() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("in", 2, 2); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__15() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Loop.mk", 7, 7); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__16() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__15; +x_2 = l_String_toSubstring_x27(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__17() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Loop", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__18() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mk", 2, 2); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__19() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__17; +x_2 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__18; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__20() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemRepeat_____closed__1; +x_2 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__17; +x_3 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__18; +x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__21() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__20; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__22() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__20; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__23() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__22; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__24() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__21; +x_2 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__23; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__25() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("do", 2, 2); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; uint8_t x_5; +x_4 = l_Lean_doElemRepeat_____closed__3; +lean_inc(x_1); +x_5 = l_Lean_Syntax_isOfKind(x_1, x_4); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; +lean_dec(x_2); +lean_dec(x_1); +x_6 = lean_box(1); +x_7 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_7, 0, x_6); +lean_ctor_set(x_7, 1, x_3); +return x_7; +} +else +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_8 = lean_unsigned_to_nat(1u); +x_9 = l_Lean_Syntax_getArg(x_1, x_8); +lean_dec(x_1); +x_10 = lean_ctor_get(x_2, 5); +lean_inc(x_10); +x_11 = 0; +x_12 = l_Lean_SourceInfo_fromRef(x_10, x_11); +lean_dec(x_10); +x_13 = lean_ctor_get(x_2, 2); +lean_inc(x_13); +x_14 = lean_ctor_get(x_2, 1); +lean_inc(x_14); +lean_dec(x_2); +x_15 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__5; +lean_inc(x_12); +x_16 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_16, 0, x_12); +lean_ctor_set(x_16, 1, x_15); +x_17 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__7; +x_18 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__10; +lean_inc(x_12); +x_19 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_19, 0, x_12); +lean_ctor_set(x_19, 1, x_17); +lean_ctor_set(x_19, 2, x_18); +x_20 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__13; +lean_inc(x_12); +x_21 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_21, 0, x_12); +lean_ctor_set(x_21, 1, x_20); +x_22 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__12; +lean_inc(x_12); +x_23 = l_Lean_Syntax_node1(x_12, x_22, x_21); +x_24 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__14; +lean_inc(x_12); +x_25 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_25, 0, x_12); +lean_ctor_set(x_25, 1, x_24); +x_26 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__19; +x_27 = l_Lean_addMacroScope(x_14, x_26, x_13); +x_28 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__16; +x_29 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__24; +lean_inc(x_12); +x_30 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_30, 0, x_12); +lean_ctor_set(x_30, 1, x_28); +lean_ctor_set(x_30, 2, x_27); +lean_ctor_set(x_30, 3, x_29); +x_31 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__9; +lean_inc(x_12); +x_32 = l_Lean_Syntax_node4(x_12, x_31, x_19, x_23, x_25, x_30); +lean_inc(x_12); +x_33 = l_Lean_Syntax_node1(x_12, x_17, x_32); +x_34 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__25; +lean_inc(x_12); +x_35 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_35, 0, x_12); +lean_ctor_set(x_35, 1, x_34); +x_36 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__4; +x_37 = l_Lean_Syntax_node4(x_12, x_36, x_16, x_33, x_35, x_9); +x_38 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_38, 0, x_37); +lean_ctor_set(x_38, 1, x_3); +return x_38; +} +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("doElemWhile_:_Do_", 17, 17); +return x_1; +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_doElemRepeat_____closed__1; +x_2 = l_Lean_doElemWhile___x3a__Do_____closed__1; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("while ", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_doElemWhile___x3a__Do_____closed__3; +x_2 = lean_alloc_ctor(5, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("ident", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_doElemWhile___x3a__Do_____closed__5; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_doElemWhile___x3a__Do_____closed__6; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemRepeat_____closed__5; +x_2 = l_Lean_doElemWhile___x3a__Do_____closed__4; +x_3 = l_Lean_doElemWhile___x3a__Do_____closed__7; +x_4 = lean_alloc_ctor(2, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__9() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" : ", 3, 3); +return x_1; +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_doElemWhile___x3a__Do_____closed__9; +x_2 = lean_alloc_ctor(5, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__11() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemRepeat_____closed__5; +x_2 = l_Lean_doElemWhile___x3a__Do_____closed__8; +x_3 = l_Lean_doElemWhile___x3a__Do_____closed__10; +x_4 = lean_alloc_ctor(2, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__12() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("termBeforeDo", 12, 12); +return x_1; +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__13() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_doElemWhile___x3a__Do_____closed__12; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__14() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_doElemWhile___x3a__Do_____closed__13; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__15() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemRepeat_____closed__5; +x_2 = l_Lean_doElemWhile___x3a__Do_____closed__11; +x_3 = l_Lean_doElemWhile___x3a__Do_____closed__14; +x_4 = lean_alloc_ctor(2, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__16() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" do ", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__17() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_doElemWhile___x3a__Do_____closed__16; +x_2 = lean_alloc_ctor(5, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__18() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemRepeat_____closed__5; +x_2 = l_Lean_doElemWhile___x3a__Do_____closed__15; +x_3 = l_Lean_doElemWhile___x3a__Do_____closed__17; +x_4 = lean_alloc_ctor(2, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__19() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemRepeat_____closed__5; +x_2 = l_Lean_doElemWhile___x3a__Do_____closed__18; +x_3 = l_Lean_doElemRepeat_____closed__10; +x_4 = lean_alloc_ctor(2, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__20() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemWhile___x3a__Do_____closed__2; +x_2 = lean_unsigned_to_nat(1022u); +x_3 = l_Lean_doElemWhile___x3a__Do_____closed__19; +x_4 = lean_alloc_ctor(3, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do__() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_doElemWhile___x3a__Do_____closed__20; +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("repeat", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("doSeqIndent", 11, 11); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_doElemRepeat_____closed__1; +x_2 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__1; +x_3 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__2; +x_4 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__2; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("doSeqItem", 9, 9); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_doElemRepeat_____closed__1; +x_2 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__1; +x_3 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__2; +x_4 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__4; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("doIf", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_doElemRepeat_____closed__1; +x_2 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__1; +x_3 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__2; +x_4 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__6; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("if", 2, 2); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__9() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("doIfProp", 8, 8); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_doElemRepeat_____closed__1; +x_2 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__1; +x_3 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__2; +x_4 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__9; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(":", 1, 1); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__12() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("then", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__13() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("else", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__14() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("doBreak", 7, 7); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__15() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_doElemRepeat_____closed__1; +x_2 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__1; +x_3 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__2; +x_4 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__14; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__16() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("break", 5, 5); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; uint8_t x_5; +x_4 = l_Lean_doElemWhile___x3a__Do_____closed__2; +lean_inc(x_1); +x_5 = l_Lean_Syntax_isOfKind(x_1, x_4); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; +lean_dec(x_1); +x_6 = lean_box(1); +x_7 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_7, 0, x_6); +lean_ctor_set(x_7, 1, x_3); +return x_7; +} +else +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_8 = lean_unsigned_to_nat(1u); +x_9 = l_Lean_Syntax_getArg(x_1, x_8); +x_10 = lean_unsigned_to_nat(3u); +x_11 = l_Lean_Syntax_getArg(x_1, x_10); +x_12 = lean_unsigned_to_nat(5u); +x_13 = l_Lean_Syntax_getArg(x_1, x_12); +lean_dec(x_1); +x_14 = lean_ctor_get(x_2, 5); +x_15 = 0; +x_16 = l_Lean_SourceInfo_fromRef(x_14, x_15); +x_17 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1; +lean_inc(x_16); +x_18 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_18, 0, x_16); +lean_ctor_set(x_18, 1, x_17); +x_19 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8; +lean_inc(x_16); +x_20 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_20, 0, x_16); +lean_ctor_set(x_20, 1, x_19); +x_21 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11; +lean_inc(x_16); +x_22 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_22, 0, x_16); +lean_ctor_set(x_22, 1, x_21); +x_23 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__7; +lean_inc(x_16); +x_24 = l_Lean_Syntax_node2(x_16, x_23, x_9, x_22); +x_25 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10; +lean_inc(x_16); +x_26 = l_Lean_Syntax_node2(x_16, x_25, x_24, x_11); +x_27 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__12; +lean_inc(x_16); +x_28 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_28, 0, x_16); +lean_ctor_set(x_28, 1, x_27); +x_29 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__10; +lean_inc(x_16); +x_30 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_30, 0, x_16); +lean_ctor_set(x_30, 1, x_23); +lean_ctor_set(x_30, 2, x_29); +x_31 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__13; +lean_inc(x_16); +x_32 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_32, 0, x_16); +lean_ctor_set(x_32, 1, x_31); +x_33 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__16; +lean_inc(x_16); +x_34 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_34, 0, x_16); +lean_ctor_set(x_34, 1, x_33); +x_35 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__15; +lean_inc(x_16); +x_36 = l_Lean_Syntax_node1(x_16, x_35, x_34); +x_37 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5; +lean_inc(x_30); +lean_inc(x_16); +x_38 = l_Lean_Syntax_node2(x_16, x_37, x_36, x_30); +lean_inc(x_16); +x_39 = l_Lean_Syntax_node1(x_16, x_23, x_38); +x_40 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3; +lean_inc(x_16); +x_41 = l_Lean_Syntax_node1(x_16, x_40, x_39); +lean_inc(x_16); +x_42 = l_Lean_Syntax_node2(x_16, x_23, x_32, x_41); +x_43 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7; +lean_inc(x_30); +lean_inc(x_16); +x_44 = l_Lean_Syntax_node6(x_16, x_43, x_20, x_26, x_28, x_13, x_30, x_42); +lean_inc(x_16); +x_45 = l_Lean_Syntax_node2(x_16, x_37, x_44, x_30); +lean_inc(x_16); +x_46 = l_Lean_Syntax_node1(x_16, x_23, x_45); +lean_inc(x_16); +x_47 = l_Lean_Syntax_node1(x_16, x_40, x_46); +x_48 = l_Lean_doElemRepeat_____closed__3; +x_49 = l_Lean_Syntax_node2(x_16, x_48, x_18, x_47); +x_50 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_50, 0, x_49); +lean_ctor_set(x_50, 1, x_3); +return x_50; +} +} +} +LEAN_EXPORT lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1(x_1, x_2, x_3); +lean_dec(x_2); +return x_4; +} +} +static lean_object* _init_l_Lean_doElemWhile__Do_____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("doElemWhile_Do_", 15, 15); +return x_1; +} +} +static lean_object* _init_l_Lean_doElemWhile__Do_____closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_doElemRepeat_____closed__1; +x_2 = l_Lean_doElemWhile__Do_____closed__1; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_doElemWhile__Do_____closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemRepeat_____closed__5; +x_2 = l_Lean_doElemWhile___x3a__Do_____closed__4; +x_3 = l_Lean_doElemWhile___x3a__Do_____closed__14; +x_4 = lean_alloc_ctor(2, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_doElemWhile__Do_____closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemRepeat_____closed__5; +x_2 = l_Lean_doElemWhile__Do_____closed__3; +x_3 = l_Lean_doElemWhile___x3a__Do_____closed__17; +x_4 = lean_alloc_ctor(2, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_doElemWhile__Do_____closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemRepeat_____closed__5; +x_2 = l_Lean_doElemWhile__Do_____closed__4; +x_3 = l_Lean_doElemRepeat_____closed__10; +x_4 = lean_alloc_ctor(2, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_doElemWhile__Do_____closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemWhile__Do_____closed__2; +x_2 = lean_unsigned_to_nat(1022u); +x_3 = l_Lean_doElemWhile__Do_____closed__5; +x_4 = lean_alloc_ctor(3, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_doElemWhile__Do__() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_doElemWhile__Do_____closed__6; +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile__Do____1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; uint8_t x_5; +x_4 = l_Lean_doElemWhile__Do_____closed__2; +lean_inc(x_1); +x_5 = l_Lean_Syntax_isOfKind(x_1, x_4); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; +lean_dec(x_1); +x_6 = lean_box(1); +x_7 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_7, 0, x_6); +lean_ctor_set(x_7, 1, x_3); +return x_7; +} +else +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_8 = lean_unsigned_to_nat(1u); +x_9 = l_Lean_Syntax_getArg(x_1, x_8); +x_10 = lean_unsigned_to_nat(3u); +x_11 = l_Lean_Syntax_getArg(x_1, x_10); +lean_dec(x_1); +x_12 = lean_ctor_get(x_2, 5); +x_13 = 0; +x_14 = l_Lean_SourceInfo_fromRef(x_12, x_13); +x_15 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1; +lean_inc(x_14); +x_16 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_16, 0, x_14); +lean_ctor_set(x_16, 1, x_15); +x_17 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8; +lean_inc(x_14); +x_18 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_18, 0, x_14); +lean_ctor_set(x_18, 1, x_17); +x_19 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__7; +x_20 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__10; +lean_inc(x_14); +x_21 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_21, 0, x_14); +lean_ctor_set(x_21, 1, x_19); +lean_ctor_set(x_21, 2, x_20); +x_22 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10; +lean_inc(x_21); +lean_inc(x_14); +x_23 = l_Lean_Syntax_node2(x_14, x_22, x_21, x_9); +x_24 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__12; +lean_inc(x_14); +x_25 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_25, 0, x_14); +lean_ctor_set(x_25, 1, x_24); +x_26 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__13; +lean_inc(x_14); +x_27 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_27, 0, x_14); +lean_ctor_set(x_27, 1, x_26); +x_28 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__16; +lean_inc(x_14); +x_29 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_29, 0, x_14); +lean_ctor_set(x_29, 1, x_28); +x_30 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__15; +lean_inc(x_14); +x_31 = l_Lean_Syntax_node1(x_14, x_30, x_29); +x_32 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5; +lean_inc(x_21); +lean_inc(x_14); +x_33 = l_Lean_Syntax_node2(x_14, x_32, x_31, x_21); +lean_inc(x_14); +x_34 = l_Lean_Syntax_node1(x_14, x_19, x_33); +x_35 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3; +lean_inc(x_14); +x_36 = l_Lean_Syntax_node1(x_14, x_35, x_34); +lean_inc(x_14); +x_37 = l_Lean_Syntax_node2(x_14, x_19, x_27, x_36); +x_38 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7; +lean_inc(x_21); +lean_inc(x_14); +x_39 = l_Lean_Syntax_node6(x_14, x_38, x_18, x_23, x_25, x_11, x_21, x_37); +lean_inc(x_14); +x_40 = l_Lean_Syntax_node2(x_14, x_32, x_39, x_21); +lean_inc(x_14); +x_41 = l_Lean_Syntax_node1(x_14, x_19, x_40); +lean_inc(x_14); +x_42 = l_Lean_Syntax_node1(x_14, x_35, x_41); +x_43 = l_Lean_doElemRepeat_____closed__3; +x_44 = l_Lean_Syntax_node2(x_14, x_43, x_16, x_42); +x_45 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_45, 0, x_44); +lean_ctor_set(x_45, 1, x_3); +return x_45; +} +} +} +LEAN_EXPORT lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile__Do____1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile__Do____1(x_1, x_2, x_3); +lean_dec(x_2); +return x_4; +} +} +static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("doElemRepeat__Until_", 20, 20); +return x_1; +} +} +static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_doElemRepeat_____closed__1; +x_2 = l_Lean_doElemRepeat____Until_____closed__1; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("ppDedent", 8, 8); +return x_1; +} +} +static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_doElemRepeat____Until_____closed__3; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("ppLine", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_doElemRepeat____Until_____closed__5; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_doElemRepeat____Until_____closed__6; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_doElemRepeat____Until_____closed__4; +x_2 = l_Lean_doElemRepeat____Until_____closed__7; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__9() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemRepeat_____closed__5; +x_2 = l_Lean_doElemRepeat_____closed__11; +x_3 = l_Lean_doElemRepeat____Until_____closed__8; +x_4 = lean_alloc_ctor(2, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__10() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("until ", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__11() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_doElemRepeat____Until_____closed__10; +x_2 = lean_alloc_ctor(5, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__12() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemRepeat_____closed__5; +x_2 = l_Lean_doElemRepeat____Until_____closed__9; +x_3 = l_Lean_doElemRepeat____Until_____closed__11; +x_4 = lean_alloc_ctor(2, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__13() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("term", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__14() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_doElemRepeat____Until_____closed__13; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__15() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_doElemRepeat____Until_____closed__14; +x_2 = lean_unsigned_to_nat(0u); +x_3 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__16() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemRepeat_____closed__5; +x_2 = l_Lean_doElemRepeat____Until_____closed__12; +x_3 = l_Lean_doElemRepeat____Until_____closed__15; +x_4 = lean_alloc_ctor(2, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__17() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemRepeat____Until_____closed__2; +x_2 = lean_unsigned_to_nat(1022u); +x_3 = l_Lean_doElemRepeat____Until_____closed__16; +x_4 = lean_alloc_ctor(3, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_doElemRepeat____Until__() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_doElemRepeat____Until_____closed__17; +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("doNested", 8, 8); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_doElemRepeat_____closed__1; +x_2 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__1; +x_3 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__2; +x_4 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___closed__1; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(";", 1, 1); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; uint8_t x_5; +x_4 = l_Lean_doElemRepeat____Until_____closed__2; +lean_inc(x_1); +x_5 = l_Lean_Syntax_isOfKind(x_1, x_4); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; +lean_dec(x_1); +x_6 = lean_box(1); +x_7 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_7, 0, x_6); +lean_ctor_set(x_7, 1, x_3); +return x_7; +} +else +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_8 = lean_unsigned_to_nat(1u); +x_9 = l_Lean_Syntax_getArg(x_1, x_8); +x_10 = lean_unsigned_to_nat(3u); +x_11 = l_Lean_Syntax_getArg(x_1, x_10); +lean_dec(x_1); +x_12 = lean_ctor_get(x_2, 5); +x_13 = 0; +x_14 = l_Lean_SourceInfo_fromRef(x_12, x_13); +x_15 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1; +lean_inc(x_14); +x_16 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_16, 0, x_14); +lean_ctor_set(x_16, 1, x_15); +x_17 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__25; +lean_inc(x_14); +x_18 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_18, 0, x_14); +lean_ctor_set(x_18, 1, x_17); +x_19 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___closed__2; +lean_inc(x_14); +x_20 = l_Lean_Syntax_node2(x_14, x_19, x_18, x_9); +x_21 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___closed__3; +lean_inc(x_14); +x_22 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_22, 0, x_14); +lean_ctor_set(x_22, 1, x_21); +x_23 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__7; +lean_inc(x_14); +x_24 = l_Lean_Syntax_node1(x_14, x_23, x_22); +x_25 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5; +lean_inc(x_14); +x_26 = l_Lean_Syntax_node2(x_14, x_25, x_20, x_24); +x_27 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8; +lean_inc(x_14); +x_28 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_28, 0, x_14); +lean_ctor_set(x_28, 1, x_27); +x_29 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__10; +lean_inc(x_14); +x_30 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_30, 0, x_14); +lean_ctor_set(x_30, 1, x_23); +lean_ctor_set(x_30, 2, x_29); +x_31 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10; +lean_inc(x_30); +lean_inc(x_14); +x_32 = l_Lean_Syntax_node2(x_14, x_31, x_30, x_11); +x_33 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__12; +lean_inc(x_14); +x_34 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_34, 0, x_14); +lean_ctor_set(x_34, 1, x_33); +x_35 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__16; +lean_inc(x_14); +x_36 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_36, 0, x_14); +lean_ctor_set(x_36, 1, x_35); +x_37 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__15; +lean_inc(x_14); +x_38 = l_Lean_Syntax_node1(x_14, x_37, x_36); +lean_inc(x_30); +lean_inc(x_14); +x_39 = l_Lean_Syntax_node2(x_14, x_25, x_38, x_30); +lean_inc(x_14); +x_40 = l_Lean_Syntax_node1(x_14, x_23, x_39); +x_41 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3; +lean_inc(x_14); +x_42 = l_Lean_Syntax_node1(x_14, x_41, x_40); +x_43 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7; +lean_inc_n(x_30, 2); +lean_inc(x_14); +x_44 = l_Lean_Syntax_node6(x_14, x_43, x_28, x_32, x_34, x_42, x_30, x_30); +lean_inc(x_14); +x_45 = l_Lean_Syntax_node2(x_14, x_25, x_44, x_30); +lean_inc(x_14); +x_46 = l_Lean_Syntax_node2(x_14, x_23, x_26, x_45); +lean_inc(x_14); +x_47 = l_Lean_Syntax_node1(x_14, x_41, x_46); +x_48 = l_Lean_doElemRepeat_____closed__3; +x_49 = l_Lean_Syntax_node2(x_14, x_48, x_16, x_47); +x_50 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_50, 0, x_49); +lean_ctor_set(x_50, 1, x_3); +return x_50; +} +} +} +LEAN_EXPORT lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1(x_1, x_2, x_3); +lean_dec(x_2); +return x_4; +} +} +lean_object* initialize_Init_Core(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Init_While(uint8_t builtin, lean_object* w) { +lean_object * res; +if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); +_G_initialized = true; +res = initialize_Init_Core(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +l_Lean_doElemRepeat_____closed__1 = _init_l_Lean_doElemRepeat_____closed__1(); +lean_mark_persistent(l_Lean_doElemRepeat_____closed__1); +l_Lean_doElemRepeat_____closed__2 = _init_l_Lean_doElemRepeat_____closed__2(); +lean_mark_persistent(l_Lean_doElemRepeat_____closed__2); +l_Lean_doElemRepeat_____closed__3 = _init_l_Lean_doElemRepeat_____closed__3(); +lean_mark_persistent(l_Lean_doElemRepeat_____closed__3); +l_Lean_doElemRepeat_____closed__4 = _init_l_Lean_doElemRepeat_____closed__4(); +lean_mark_persistent(l_Lean_doElemRepeat_____closed__4); +l_Lean_doElemRepeat_____closed__5 = _init_l_Lean_doElemRepeat_____closed__5(); +lean_mark_persistent(l_Lean_doElemRepeat_____closed__5); +l_Lean_doElemRepeat_____closed__6 = _init_l_Lean_doElemRepeat_____closed__6(); +lean_mark_persistent(l_Lean_doElemRepeat_____closed__6); +l_Lean_doElemRepeat_____closed__7 = _init_l_Lean_doElemRepeat_____closed__7(); +lean_mark_persistent(l_Lean_doElemRepeat_____closed__7); +l_Lean_doElemRepeat_____closed__8 = _init_l_Lean_doElemRepeat_____closed__8(); +lean_mark_persistent(l_Lean_doElemRepeat_____closed__8); +l_Lean_doElemRepeat_____closed__9 = _init_l_Lean_doElemRepeat_____closed__9(); +lean_mark_persistent(l_Lean_doElemRepeat_____closed__9); +l_Lean_doElemRepeat_____closed__10 = _init_l_Lean_doElemRepeat_____closed__10(); +lean_mark_persistent(l_Lean_doElemRepeat_____closed__10); +l_Lean_doElemRepeat_____closed__11 = _init_l_Lean_doElemRepeat_____closed__11(); +lean_mark_persistent(l_Lean_doElemRepeat_____closed__11); +l_Lean_doElemRepeat_____closed__12 = _init_l_Lean_doElemRepeat_____closed__12(); +lean_mark_persistent(l_Lean_doElemRepeat_____closed__12); +l_Lean_doElemRepeat__ = _init_l_Lean_doElemRepeat__(); +lean_mark_persistent(l_Lean_doElemRepeat__); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__1 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__1(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__1); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__2 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__2(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__2); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__3 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__3(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__3); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__4 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__4(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__4); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__5 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__5(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__5); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__6 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__6(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__6); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__7 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__7(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__7); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__8 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__8(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__8); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__9 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__9(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__9); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__10 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__10(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__10); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__11 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__11(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__11); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__12 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__12(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__12); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__13 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__13(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__13); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__14 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__14(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__14); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__15 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__15(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__15); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__16 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__16(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__16); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__17 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__17(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__17); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__18 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__18(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__18); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__19 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__19(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__19); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__20 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__20(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__20); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__21 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__21(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__21); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__22 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__22(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__22); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__23 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__23(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__23); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__24 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__24(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__24); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__25 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__25(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__25); +l_Lean_doElemWhile___x3a__Do_____closed__1 = _init_l_Lean_doElemWhile___x3a__Do_____closed__1(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__1); +l_Lean_doElemWhile___x3a__Do_____closed__2 = _init_l_Lean_doElemWhile___x3a__Do_____closed__2(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__2); +l_Lean_doElemWhile___x3a__Do_____closed__3 = _init_l_Lean_doElemWhile___x3a__Do_____closed__3(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__3); +l_Lean_doElemWhile___x3a__Do_____closed__4 = _init_l_Lean_doElemWhile___x3a__Do_____closed__4(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__4); +l_Lean_doElemWhile___x3a__Do_____closed__5 = _init_l_Lean_doElemWhile___x3a__Do_____closed__5(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__5); +l_Lean_doElemWhile___x3a__Do_____closed__6 = _init_l_Lean_doElemWhile___x3a__Do_____closed__6(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__6); +l_Lean_doElemWhile___x3a__Do_____closed__7 = _init_l_Lean_doElemWhile___x3a__Do_____closed__7(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__7); +l_Lean_doElemWhile___x3a__Do_____closed__8 = _init_l_Lean_doElemWhile___x3a__Do_____closed__8(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__8); +l_Lean_doElemWhile___x3a__Do_____closed__9 = _init_l_Lean_doElemWhile___x3a__Do_____closed__9(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__9); +l_Lean_doElemWhile___x3a__Do_____closed__10 = _init_l_Lean_doElemWhile___x3a__Do_____closed__10(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__10); +l_Lean_doElemWhile___x3a__Do_____closed__11 = _init_l_Lean_doElemWhile___x3a__Do_____closed__11(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__11); +l_Lean_doElemWhile___x3a__Do_____closed__12 = _init_l_Lean_doElemWhile___x3a__Do_____closed__12(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__12); +l_Lean_doElemWhile___x3a__Do_____closed__13 = _init_l_Lean_doElemWhile___x3a__Do_____closed__13(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__13); +l_Lean_doElemWhile___x3a__Do_____closed__14 = _init_l_Lean_doElemWhile___x3a__Do_____closed__14(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__14); +l_Lean_doElemWhile___x3a__Do_____closed__15 = _init_l_Lean_doElemWhile___x3a__Do_____closed__15(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__15); +l_Lean_doElemWhile___x3a__Do_____closed__16 = _init_l_Lean_doElemWhile___x3a__Do_____closed__16(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__16); +l_Lean_doElemWhile___x3a__Do_____closed__17 = _init_l_Lean_doElemWhile___x3a__Do_____closed__17(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__17); +l_Lean_doElemWhile___x3a__Do_____closed__18 = _init_l_Lean_doElemWhile___x3a__Do_____closed__18(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__18); +l_Lean_doElemWhile___x3a__Do_____closed__19 = _init_l_Lean_doElemWhile___x3a__Do_____closed__19(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__19); +l_Lean_doElemWhile___x3a__Do_____closed__20 = _init_l_Lean_doElemWhile___x3a__Do_____closed__20(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__20); +l_Lean_doElemWhile___x3a__Do__ = _init_l_Lean_doElemWhile___x3a__Do__(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do__); +l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1); +l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__2 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__2(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__2); +l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3); +l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__4 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__4(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__4); +l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5); +l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__6 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__6(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__6); +l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7); +l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8); +l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__9 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__9(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__9); +l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10); +l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11); +l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__12 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__12(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__12); +l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__13 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__13(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__13); +l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__14 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__14(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__14); +l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__15 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__15(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__15); +l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__16 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__16(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__16); +l_Lean_doElemWhile__Do_____closed__1 = _init_l_Lean_doElemWhile__Do_____closed__1(); +lean_mark_persistent(l_Lean_doElemWhile__Do_____closed__1); +l_Lean_doElemWhile__Do_____closed__2 = _init_l_Lean_doElemWhile__Do_____closed__2(); +lean_mark_persistent(l_Lean_doElemWhile__Do_____closed__2); +l_Lean_doElemWhile__Do_____closed__3 = _init_l_Lean_doElemWhile__Do_____closed__3(); +lean_mark_persistent(l_Lean_doElemWhile__Do_____closed__3); +l_Lean_doElemWhile__Do_____closed__4 = _init_l_Lean_doElemWhile__Do_____closed__4(); +lean_mark_persistent(l_Lean_doElemWhile__Do_____closed__4); +l_Lean_doElemWhile__Do_____closed__5 = _init_l_Lean_doElemWhile__Do_____closed__5(); +lean_mark_persistent(l_Lean_doElemWhile__Do_____closed__5); +l_Lean_doElemWhile__Do_____closed__6 = _init_l_Lean_doElemWhile__Do_____closed__6(); +lean_mark_persistent(l_Lean_doElemWhile__Do_____closed__6); +l_Lean_doElemWhile__Do__ = _init_l_Lean_doElemWhile__Do__(); +lean_mark_persistent(l_Lean_doElemWhile__Do__); +l_Lean_doElemRepeat____Until_____closed__1 = _init_l_Lean_doElemRepeat____Until_____closed__1(); +lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__1); +l_Lean_doElemRepeat____Until_____closed__2 = _init_l_Lean_doElemRepeat____Until_____closed__2(); +lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__2); +l_Lean_doElemRepeat____Until_____closed__3 = _init_l_Lean_doElemRepeat____Until_____closed__3(); +lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__3); +l_Lean_doElemRepeat____Until_____closed__4 = _init_l_Lean_doElemRepeat____Until_____closed__4(); +lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__4); +l_Lean_doElemRepeat____Until_____closed__5 = _init_l_Lean_doElemRepeat____Until_____closed__5(); +lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__5); +l_Lean_doElemRepeat____Until_____closed__6 = _init_l_Lean_doElemRepeat____Until_____closed__6(); +lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__6); +l_Lean_doElemRepeat____Until_____closed__7 = _init_l_Lean_doElemRepeat____Until_____closed__7(); +lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__7); +l_Lean_doElemRepeat____Until_____closed__8 = _init_l_Lean_doElemRepeat____Until_____closed__8(); +lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__8); +l_Lean_doElemRepeat____Until_____closed__9 = _init_l_Lean_doElemRepeat____Until_____closed__9(); +lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__9); +l_Lean_doElemRepeat____Until_____closed__10 = _init_l_Lean_doElemRepeat____Until_____closed__10(); +lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__10); +l_Lean_doElemRepeat____Until_____closed__11 = _init_l_Lean_doElemRepeat____Until_____closed__11(); +lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__11); +l_Lean_doElemRepeat____Until_____closed__12 = _init_l_Lean_doElemRepeat____Until_____closed__12(); +lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__12); +l_Lean_doElemRepeat____Until_____closed__13 = _init_l_Lean_doElemRepeat____Until_____closed__13(); +lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__13); +l_Lean_doElemRepeat____Until_____closed__14 = _init_l_Lean_doElemRepeat____Until_____closed__14(); +lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__14); +l_Lean_doElemRepeat____Until_____closed__15 = _init_l_Lean_doElemRepeat____Until_____closed__15(); +lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__15); +l_Lean_doElemRepeat____Until_____closed__16 = _init_l_Lean_doElemRepeat____Until_____closed__16(); +lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__16); +l_Lean_doElemRepeat____Until_____closed__17 = _init_l_Lean_doElemRepeat____Until_____closed__17(); +lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__17); +l_Lean_doElemRepeat____Until__ = _init_l_Lean_doElemRepeat____Until__(); +lean_mark_persistent(l_Lean_doElemRepeat____Until__); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___closed__1 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___closed__1(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___closed__1); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___closed__2 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___closed__2(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___closed__2); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___closed__3 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___closed__3(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___closed__3); +return lean_io_result_mk_ok(lean_box(0)); +} +#ifdef __cplusplus +} +#endif diff --git a/stage0/stdlib/Lake/Build/Common.c b/stage0/stdlib/Lake/Build/Common.c index d8c313ce6108..71ec0bf8bbec 100644 --- a/stage0/stdlib/Lake/Build/Common.c +++ b/stage0/stdlib/Lake/Build/Common.c @@ -190,6 +190,7 @@ lean_object* l_Array_extract___rarg(lean_object*, lean_object*, lean_object*); lean_object* l_Substring_nextn(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_buildFileAfterDep(lean_object*); LEAN_EXPORT lean_object* l_IO_withStderr___at_Lake_buildFileAfterDep___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(lean_object*, lean_object*); static lean_object* l_Lake_computeDynlibOfShared___lambda__2___closed__7; lean_object* l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_computeDynlibOfShared(lean_object*, lean_object*, lean_object*); @@ -219,7 +220,6 @@ lean_object* l_Substring_takeRightWhileAux___at_Substring_trimRight___spec__1(le LEAN_EXPORT lean_object* l_Lake_buildUnlessUpToDate_x3f___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_buildO___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_buildLeanSharedLibOfStatic___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_List_bindTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_computeDynlibOfShared___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_computeDynlibOfShared___lambda__2___closed__3; lean_object* l_Array_mapMUnsafe_map___at_Lake_instFromJsonLog___spec__1(size_t, size_t, lean_object*); @@ -393,7 +393,7 @@ x_19 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_19, 0, x_9); lean_ctor_set(x_19, 1, x_18); x_20 = l___private_Lake_Build_Common_0__Lake_toJsonBuildMetadata____x40_Lake_Build_Common___hyg_31____closed__3; -x_21 = l_List_bindTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(x_19, x_20); +x_21 = l_List_flatMapTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(x_19, x_20); x_22 = l_Lean_Json_mkObj(x_21); return x_22; } diff --git a/stage0/stdlib/Lake/Build/Facets.c b/stage0/stdlib/Lake/Build/Facets.c index 52ad5de8b9f1..7bfd127b6ba6 100644 --- a/stage0/stdlib/Lake/Build/Facets.c +++ b/stage0/stdlib/Lake/Build/Facets.c @@ -15,29 +15,35 @@ extern "C" { #endif static lean_object* l_Lake_Module_cFacet___closed__2; static lean_object* l_Lake_Module_coNoExportFacet___closed__2; +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__7; lean_object* l_Lean_Name_reprPrec(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_Module_coExportFacet; -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__9; static lean_object* l_Lake_Module_ileanFacet___closed__2; -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__2; LEAN_EXPORT lean_object* l_Lake_instCoeDepNameModuleFacetOfFamilyOutModuleData___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_Package_reservoirBarrelFacet___closed__1; LEAN_EXPORT lean_object* l_Lake_instReprModuleFacet___boxed(lean_object*, lean_object*); +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__17; static lean_object* l_Lake_ExternLib_staticFacet___closed__2; static lean_object* l_Lake_ExternLib_dynlibFacet___closed__2; static lean_object* l_Lake_Package_gitHubReleaseFacet___closed__1; static lean_object* l_Lake_Module_oFacet___closed__1; +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__18; +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__2; LEAN_EXPORT lean_object* l_Lake_ExternLib_sharedFacet; +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__9; +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__15; +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__12; LEAN_EXPORT lean_object* l_Lake_Module_cFacet; static lean_object* l_Lake_ExternLib_staticFacet___closed__1; LEAN_EXPORT lean_object* l_Lake_ExternLib_dynlibFacet; static lean_object* l_Lake_Package_extraDepFacet___closed__1; -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__13; -LEAN_EXPORT lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_Module_ileanFacet; static lean_object* l_Lake_Module_leanArtsFacet___closed__1; +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__4; static lean_object* l_Lake_Package_gitHubReleaseFacet___closed__2; LEAN_EXPORT lean_object* l_Lake_Module_depsFacet; +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__10; LEAN_EXPORT lean_object* l_Lake_LeanLib_extraDepFacet; static lean_object* l_Lake_Module_bcFacet___closed__2; LEAN_EXPORT lean_object* l_Lake_Dynlib_dir_x3f(lean_object*); @@ -45,32 +51,31 @@ static lean_object* l_Lake_Module_ileanFacet___closed__1; LEAN_EXPORT lean_object* l_Lake_Package_gitHubReleaseFacet; LEAN_EXPORT lean_object* l_Lake_Module_coNoExportFacet; static lean_object* l_Lake_instReprModuleFacet___closed__1; -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__5; static lean_object* l_Lake_Package_reservoirBarrelFacet___closed__2; lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__11; -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__17; LEAN_EXPORT lean_object* l_Lake_LeanExe_exeFacet; -LEAN_EXPORT lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___boxed(lean_object*, lean_object*); static lean_object* l_Lake_Module_bcoFacet___closed__1; +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__8; static lean_object* l_Lake_Module_oleanFacet___closed__2; static lean_object* l_Lake_LeanLib_staticFacet___closed__1; static lean_object* l_Lake_LeanLib_sharedFacet___closed__2; -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__19; +LEAN_EXPORT lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____boxed(lean_object*, lean_object*); lean_object* lean_nat_to_int(lean_object*); static lean_object* l_Lake_LeanLib_sharedFacet___closed__1; static lean_object* l_Lake_Package_buildCacheFacet___closed__2; +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__14; LEAN_EXPORT lean_object* l_Lake_LeanLib_leanArtsFacet; LEAN_EXPORT lean_object* l_Lake_Module_leanArtsFacet; -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__16; +LEAN_EXPORT lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66_(lean_object*, lean_object*); +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__11; static lean_object* l_Lake_Module_coExportFacet___closed__2; static lean_object* l_Lake_Module_oleanFacet___closed__1; -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__14; +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__5; +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__13; LEAN_EXPORT lean_object* l_Lake_Module_bcFacet; static lean_object* l_Lake_Package_optReservoirBarrelFacet___closed__1; -LEAN_EXPORT lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg(lean_object*, lean_object*); +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__16; lean_object* l_System_FilePath_parent(lean_object*); -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__18; static lean_object* l_Lake_Module_oExportFacet___closed__1; static lean_object* l_Lake_LeanLib_staticExportFacet___closed__1; static lean_object* l_Lake_LeanLib_staticFacet___closed__2; @@ -78,55 +83,50 @@ lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_instCoeDepNameModuleFacetOfFamilyOutModuleData(lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_Package_buildCacheFacet___closed__1; static lean_object* l_Lake_ExternLib_sharedFacet___closed__1; -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__12; static lean_object* l_Lake_LeanExe_exeFacet___closed__1; LEAN_EXPORT lean_object* l_Lake_LeanLib_staticFacet; static lean_object* l_Lake_Module_coFacet___closed__2; LEAN_EXPORT lean_object* l_Lake_Package_buildCacheFacet; -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__15; -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__10; static lean_object* l_Lake_Package_optBuildCacheFacet___closed__1; static lean_object* l_Lake_Module_depsFacet___closed__2; LEAN_EXPORT lean_object* l_Lake_LeanLib_staticExportFacet; +LEAN_EXPORT lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_Package_extraDepFacet; lean_object* lean_string_length(lean_object*); static lean_object* l_Lake_Package_optGitHubReleaseFacet___closed__2; static lean_object* l_Lake_Package_optReservoirBarrelFacet___closed__2; -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__3; static lean_object* l_Lake_Module_coNoExportFacet___closed__1; static lean_object* l_Lake_Module_leanArtsFacet___closed__2; -LEAN_EXPORT lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_Package_optGitHubReleaseFacet; lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); static lean_object* l_Lake_ExternLib_dynlibFacet___closed__1; -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__8; LEAN_EXPORT lean_object* l_Lake_Module_coFacet; static lean_object* l_Lake_Module_cFacet___closed__1; LEAN_EXPORT lean_object* l_Lake_Module_bcoFacet; LEAN_EXPORT lean_object* l_Lake_Module_oExportFacet; +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__6; +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__19; +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__1; LEAN_EXPORT lean_object* l_Lake_Package_releaseFacet; static lean_object* l_Lake_Package_optBuildCacheFacet___closed__2; LEAN_EXPORT lean_object* l_Lake_instReprModuleFacet(lean_object*, lean_object*); static lean_object* l_Lake_Module_coFacet___closed__1; static lean_object* l_Lake_Package_extraDepFacet___closed__2; LEAN_EXPORT lean_object* l_Lake_Dynlib_dir_x3f___boxed(lean_object*); -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__6; LEAN_EXPORT lean_object* l_Lake_ExternLib_staticFacet; LEAN_EXPORT lean_object* l_Lake_Module_oNoExportFacet; -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__4; LEAN_EXPORT lean_object* l_Lake_Package_reservoirBarrelFacet; LEAN_EXPORT lean_object* l_Lake_Package_optBuildCacheFacet; static lean_object* l_Lake_Package_optGitHubReleaseFacet___closed__1; static lean_object* l_Lake_Module_depsFacet___closed__1; static lean_object* l_Lake_Module_coExportFacet___closed__1; -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__1; LEAN_EXPORT lean_object* l_Lake_LeanLib_sharedFacet; +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__3; LEAN_EXPORT lean_object* l_Lake_Module_oleanFacet; static lean_object* l_Lake_Module_oNoExportFacet___closed__1; LEAN_EXPORT lean_object* l_Lake_Module_oFacet; static lean_object* l_Lake_LeanExe_exeFacet___closed__2; LEAN_EXPORT lean_object* l_Lake_Package_optReleaseFacet; -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__7; LEAN_EXPORT lean_object* l_Lake_Package_optReservoirBarrelFacet; static lean_object* l_Lake_Module_bcFacet___closed__1; LEAN_EXPORT lean_object* l_Lake_Dynlib_dir_x3f(lean_object* x_1) { @@ -147,7 +147,7 @@ lean_dec(x_1); return x_2; } } -static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__1() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__1() { _start: { lean_object* x_1; @@ -155,29 +155,29 @@ x_1 = lean_mk_string_unchecked("name", 4, 4); return x_1; } } -static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__2() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__1; +x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__1; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__3() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__2; +x_2 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__2; x_3 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__4() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__4() { _start: { lean_object* x_1; @@ -185,29 +185,29 @@ x_1 = lean_mk_string_unchecked(" := ", 4, 4); return x_1; } } -static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__5() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__5() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__4; +x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__4; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__6() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__3; -x_2 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__5; +x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__3; +x_2 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__5; x_3 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__7() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__7() { _start: { lean_object* x_1; lean_object* x_2; @@ -216,7 +216,7 @@ x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__8() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__8() { _start: { lean_object* x_1; @@ -224,17 +224,17 @@ x_1 = lean_mk_string_unchecked(",", 1, 1); return x_1; } } -static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__9() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__9() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__8; +x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__8; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__10() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__10() { _start: { lean_object* x_1; @@ -242,17 +242,17 @@ x_1 = lean_mk_string_unchecked("data_eq", 7, 7); return x_1; } } -static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__11() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__11() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__10; +x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__10; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__12() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__12() { _start: { lean_object* x_1; @@ -260,17 +260,17 @@ x_1 = lean_mk_string_unchecked("_", 1, 1); return x_1; } } -static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__13() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__13() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__12; +x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__12; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__14() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__14() { _start: { lean_object* x_1; @@ -278,35 +278,35 @@ x_1 = lean_mk_string_unchecked("{ ", 2, 2); return x_1; } } -static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__15() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__15() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__14; +x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__14; x_2 = lean_string_length(x_1); return x_2; } } -static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__16() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__16() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__15; +x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__15; x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__17() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__17() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__14; +x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__14; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__18() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__18() { _start: { lean_object* x_1; @@ -314,23 +314,23 @@ x_1 = lean_mk_string_unchecked(" }", 2, 2); return x_1; } } -static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__19() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__19() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__18; +x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__18; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; uint8_t x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; x_3 = lean_unsigned_to_nat(0u); x_4 = l_Lean_Name_reprPrec(x_1, x_3); -x_5 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__7; +x_5 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__7; x_6 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_6, 0, x_5); lean_ctor_set(x_6, 1, x_4); @@ -338,11 +338,11 @@ x_7 = 0; x_8 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_8, 0, x_6); lean_ctor_set_uint8(x_8, sizeof(void*)*1, x_7); -x_9 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__6; +x_9 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__6; x_10 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_10, 0, x_9); lean_ctor_set(x_10, 1, x_8); -x_11 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__9; +x_11 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__9; x_12 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_12, 0, x_10); lean_ctor_set(x_12, 1, x_11); @@ -350,27 +350,27 @@ x_13 = lean_box(1); x_14 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_14, 0, x_12); lean_ctor_set(x_14, 1, x_13); -x_15 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__11; +x_15 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__11; x_16 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_16, 0, x_14); lean_ctor_set(x_16, 1, x_15); -x_17 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__5; +x_17 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__5; x_18 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_18, 0, x_16); lean_ctor_set(x_18, 1, x_17); -x_19 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__13; +x_19 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__13; x_20 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_20, 0, x_18); lean_ctor_set(x_20, 1, x_19); -x_21 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__17; +x_21 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__17; x_22 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_22, 0, x_21); lean_ctor_set(x_22, 1, x_20); -x_23 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__19; +x_23 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__19; x_24 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_24, 0, x_22); lean_ctor_set(x_24, 1, x_23); -x_25 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__16; +x_25 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__16; x_26 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_26, 0, x_25); lean_ctor_set(x_26, 1, x_24); @@ -380,28 +380,28 @@ lean_ctor_set_uint8(x_27, sizeof(void*)*1, x_7); return x_27; } } -LEAN_EXPORT lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65_(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66_(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___boxed), 2, 0); +x_3 = lean_alloc_closure((void*)(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___boxed), 2, 0); return x_3; } } -LEAN_EXPORT lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg(x_1, x_2); +x_3 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg(x_1, x_2); lean_dec(x_2); return x_3; } } -LEAN_EXPORT lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65_(x_1, x_2); +x_3 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66_(x_1, x_2); lean_dec(x_2); return x_3; } @@ -410,7 +410,7 @@ static lean_object* _init_l_Lake_instReprModuleFacet___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___boxed), 2, 0); return x_1; } } @@ -1152,44 +1152,44 @@ lean_dec_ref(res); res = initialize_Lake_Build_Data(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__1 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__1(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__1); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__2 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__2(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__2); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__3 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__3(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__3); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__4 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__4(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__4); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__5 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__5(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__5); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__6 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__6(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__6); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__7 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__7(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__7); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__8 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__8(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__8); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__9 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__9(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__9); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__10 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__10(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__10); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__11 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__11(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__11); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__12 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__12(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__12); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__13 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__13(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__13); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__14 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__14(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__14); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__15 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__15(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__15); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__16 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__16(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__16); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__17 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__17(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__17); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__18 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__18(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__18); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__19 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__19(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__19); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__1 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__1(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__1); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__2 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__2(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__2); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__3 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__3(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__3); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__4 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__4(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__4); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__5 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__5(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__5); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__6 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__6(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__6); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__7 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__7(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__7); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__8 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__8(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__8); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__9 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__9(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__9); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__10 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__10(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__10); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__11 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__11(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__11); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__12 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__12(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__12); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__13 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__13(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__13); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__14 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__14(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__14); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__15 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__15(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__15); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__16 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__16(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__16); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__17 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__17(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__17); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__18 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__18(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__18); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__19 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__19(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__19); l_Lake_instReprModuleFacet___closed__1 = _init_l_Lake_instReprModuleFacet___closed__1(); lean_mark_persistent(l_Lake_instReprModuleFacet___closed__1); l_Lake_Module_depsFacet___closed__1 = _init_l_Lake_Module_depsFacet___closed__1(); diff --git a/stage0/stdlib/Lake/Build/Fetch.c b/stage0/stdlib/Lake/Build/Fetch.c index 5b225389cf45..1fd46a9498c1 100644 --- a/stage0/stdlib/Lake/Build/Fetch.c +++ b/stage0/stdlib/Lake/Build/Fetch.c @@ -14,6 +14,7 @@ extern "C" { #endif static lean_object* l_Lake_instMonadCycleOfBuildKeyRecBuildM___closed__3; +lean_object* l_Array_take___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_registerJob___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_RecBuildM_run___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_instMonadLiftLogIORecBuildM(lean_object*); @@ -88,7 +89,6 @@ LEAN_EXPORT lean_object* l_Lake_withRegisterJob(lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); static lean_object* l_Lake_instMonadCycleOfBuildKeyRecBuildM___closed__5; LEAN_EXPORT lean_object* l_Lake_registerJob___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Array_shrink___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_buildCycleError(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_buildCycleError___rarg(lean_object*, lean_object*); lean_object* lean_task_map(lean_object*, lean_object*, lean_object*, uint8_t); @@ -6064,7 +6064,7 @@ lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean x_15 = lean_ctor_get(x_11, 0); x_16 = lean_ctor_get(x_11, 1); lean_inc(x_16); -x_17 = l_Array_shrink___rarg(x_16, x_8); +x_17 = l_Array_take___rarg(x_16, x_8); x_18 = lean_array_get_size(x_16); x_19 = l_Array_extract___rarg(x_16, x_8, x_18); lean_dec(x_18); @@ -6137,7 +6137,7 @@ lean_inc(x_40); lean_inc(x_39); lean_dec(x_11); lean_inc(x_40); -x_41 = l_Array_shrink___rarg(x_40, x_8); +x_41 = l_Array_take___rarg(x_40, x_8); x_42 = lean_array_get_size(x_40); x_43 = l_Array_extract___rarg(x_40, x_8, x_42); lean_dec(x_42); @@ -6218,7 +6218,7 @@ if (lean_is_exclusive(x_11)) { x_63 = lean_box(0); } lean_inc(x_62); -x_64 = l_Array_shrink___rarg(x_62, x_8); +x_64 = l_Array_take___rarg(x_62, x_8); x_65 = lean_array_get_size(x_62); x_66 = l_Array_extract___rarg(x_62, x_8, x_65); lean_dec(x_65); @@ -6309,7 +6309,7 @@ x_88 = lean_ctor_get(x_11, 1); x_89 = lean_ctor_get(x_11, 0); lean_dec(x_89); lean_inc(x_88); -x_90 = l_Array_shrink___rarg(x_88, x_8); +x_90 = l_Array_take___rarg(x_88, x_8); x_91 = lean_array_get_size(x_88); x_92 = l_Array_extract___rarg(x_88, x_8, x_91); lean_dec(x_91); @@ -6344,7 +6344,7 @@ x_102 = lean_ctor_get(x_11, 1); lean_inc(x_102); lean_dec(x_11); lean_inc(x_102); -x_103 = l_Array_shrink___rarg(x_102, x_8); +x_103 = l_Array_take___rarg(x_102, x_8); x_104 = lean_array_get_size(x_102); x_105 = l_Array_extract___rarg(x_102, x_8, x_104); lean_dec(x_104); @@ -6391,7 +6391,7 @@ if (lean_is_exclusive(x_11)) { x_118 = lean_box(0); } lean_inc(x_117); -x_119 = l_Array_shrink___rarg(x_117, x_8); +x_119 = l_Array_take___rarg(x_117, x_8); x_120 = lean_array_get_size(x_117); x_121 = l_Array_extract___rarg(x_117, x_8, x_120); lean_dec(x_120); diff --git a/stage0/stdlib/Lake/Build/Imports.c b/stage0/stdlib/Lake/Build/Imports.c index 35c1258dc398..3d88d4d40ae0 100644 --- a/stage0/stdlib/Lake/Build/Imports.c +++ b/stage0/stdlib/Lake/Build/Imports.c @@ -15,6 +15,7 @@ extern "C" { #endif LEAN_EXPORT lean_object* l_Lake_buildImportsAndDeps___lambda__8(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lake_buildImportsAndDeps___spec__8___closed__8; +lean_object* l_Array_take___rarg(lean_object*, lean_object*); lean_object* l_Lake_OrdHashSet_insert___at_Lake_Module_recParseImports___spec__2(lean_object*, lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); static lean_object* l_Lake_buildImportsAndDeps___lambda__12___closed__1; @@ -109,7 +110,6 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lake_buildImportsAndDeps_ lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_buildImportsAndDeps___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lake_BuildJob_mixArray___rarg(lean_object*); -lean_object* l_Array_shrink___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_buildImportsAndDeps___lambda__4(lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_task_map(lean_object*, lean_object*, lean_object*, uint8_t); lean_object* lean_io_bind_task(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*); @@ -5368,7 +5368,7 @@ if (x_117 == 0) lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; 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_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; x_118 = lean_ctor_get(x_110, 0); x_119 = lean_ctor_get(x_110, 1); -x_120 = l_Array_shrink___rarg(x_119, x_118); +x_120 = l_Array_take___rarg(x_119, x_118); lean_dec(x_118); x_121 = l_Array_forInUnsafe_loop___at_Lake_buildImportsAndDeps___spec__8___closed__1; x_122 = lean_string_append(x_121, x_1); @@ -5416,7 +5416,7 @@ x_140 = lean_ctor_get(x_110, 1); lean_inc(x_140); lean_inc(x_139); lean_dec(x_110); -x_141 = l_Array_shrink___rarg(x_140, x_139); +x_141 = l_Array_take___rarg(x_140, x_139); lean_dec(x_139); x_142 = l_Array_forInUnsafe_loop___at_Lake_buildImportsAndDeps___spec__8___closed__1; x_143 = lean_string_append(x_142, x_1); @@ -5476,7 +5476,7 @@ if (lean_is_exclusive(x_110)) { lean_dec_ref(x_110); x_164 = lean_box(0); } -x_165 = l_Array_shrink___rarg(x_163, x_162); +x_165 = l_Array_take___rarg(x_163, x_162); lean_dec(x_162); x_166 = l_Array_forInUnsafe_loop___at_Lake_buildImportsAndDeps___spec__8___closed__1; x_167 = lean_string_append(x_166, x_1); diff --git a/stage0/stdlib/Lake/Build/Index.c b/stage0/stdlib/Lake/Build/Index.c index 404039800d43..260b4e3ad000 100644 --- a/stage0/stdlib/Lake/Build/Index.c +++ b/stage0/stdlib/Lake/Build/Index.c @@ -46,7 +46,6 @@ static lean_object* l_Lake_ExternLib_recBuildStatic___closed__4; lean_object* l_Lake_withRegisterJob___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_EquipT_map___at_Lake_ExternLib_recBuildStatic___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_partition_loop___at_Lake_FetchM_run___spec__5___boxed(lean_object*, lean_object*, lean_object*); -uint8_t l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_325_(lean_object*, lean_object*); lean_object* l_Lake_Workspace_findLibraryFacetConfig_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_ExternLib_recBuildShared(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_EquipT_map___at_Lake_ExternLib_recBuildStatic___spec__1(lean_object*, lean_object*); @@ -84,6 +83,7 @@ lean_object* lean_array_mk(lean_object*); lean_object* lean_string_append(lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); uint8_t l_Lake_BuildKey_quickCmp(lean_object*, lean_object*); +uint8_t l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_326_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_FetchM_run(lean_object*); LEAN_EXPORT lean_object* l_Lake_mkTargetFacetBuild___boxed(lean_object*, lean_object*); lean_object* l_Lake_LeanExe_recBuildExe(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1350,7 +1350,7 @@ else lean_object* x_4; lean_object* x_5; uint8_t x_6; x_4 = lean_ctor_get(x_2, 0); x_5 = lean_ctor_get(x_2, 1); -x_6 = l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_325_(x_1, x_4); +x_6 = l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_326_(x_1, x_4); if (x_6 == 0) { x_2 = x_5; @@ -3852,7 +3852,7 @@ x_16 = lean_ctor_get(x_2, 0); x_17 = lean_ctor_get(x_2, 1); x_18 = lean_ctor_get(x_3, 0); x_19 = lean_ctor_get(x_3, 1); -x_20 = l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_325_(x_16, x_1); +x_20 = l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_326_(x_16, x_1); if (x_20 == 0) { lean_ctor_set(x_2, 1, x_18); @@ -3878,7 +3878,7 @@ x_26 = lean_ctor_get(x_3, 1); lean_inc(x_26); lean_inc(x_25); lean_dec(x_3); -x_27 = l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_325_(x_23, x_1); +x_27 = l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_326_(x_23, x_1); if (x_27 == 0) { lean_object* x_28; @@ -3923,7 +3923,7 @@ if (lean_is_exclusive(x_3)) { lean_dec_ref(x_3); x_36 = lean_box(0); } -x_37 = l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_325_(x_32, x_1); +x_37 = l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_326_(x_32, x_1); if (x_37 == 0) { lean_object* x_38; lean_object* x_39; diff --git a/stage0/stdlib/Lake/Build/Job.c b/stage0/stdlib/Lake/Build/Job.c index 91fbf83fc94c..b04606312cb5 100644 --- a/stage0/stdlib/Lake/Build/Job.c +++ b/stage0/stdlib/Lake/Build/Job.c @@ -17,6 +17,7 @@ static lean_object* l_Lake_instMonadStateOfLogJobM___closed__4; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lake_BuildJob_collectArray___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lake_BuildJob_mix___rarg___lambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lake_BuildJob_mixList___spec__2___rarg___lambda__1(lean_object*, lean_object*); +lean_object* l_Array_take___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_BuildJob_zipWith___rarg___lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_BuildJob_collectArray___rarg___boxed(lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lake_BuildJob_mixList___spec__2___rarg(lean_object*, size_t, size_t, lean_object*); @@ -301,7 +302,6 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lake_BuildJob_mixArray__ LEAN_EXPORT lean_object* l_IO_withStderr___at_Lake_BuildJob_bindSync___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_BuildJob_mixArray___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lake_instMonadLiftLakeMBuildTOfPure___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Array_shrink___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_BuildJob_instFunctor___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_Job_bindSync___rarg(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_IO_withStdout___at_Lake_Job_bindSync___spec__5(lean_object*); @@ -1978,7 +1978,7 @@ if (x_16 == 0) { lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; x_17 = lean_ctor_get(x_13, 0); -x_18 = l_Array_shrink___rarg(x_17, x_15); +x_18 = l_Array_take___rarg(x_17, x_15); lean_dec(x_15); lean_ctor_set(x_13, 0, x_18); x_19 = lean_box(0); @@ -1992,7 +1992,7 @@ x_21 = lean_ctor_get(x_13, 0); x_22 = lean_ctor_get_uint8(x_13, sizeof(void*)*1); lean_inc(x_21); lean_dec(x_13); -x_23 = l_Array_shrink___rarg(x_21, x_15); +x_23 = l_Array_take___rarg(x_21, x_15); lean_dec(x_15); x_24 = lean_alloc_ctor(0, 1, 1); lean_ctor_set(x_24, 0, x_23); diff --git a/stage0/stdlib/Lake/Build/Key.c b/stage0/stdlib/Lake/Build/Key.c index fd77dd167432..849128964e10 100644 --- a/stage0/stdlib/Lake/Build/Key.c +++ b/stage0/stdlib/Lake/Build/Key.c @@ -13,32 +13,32 @@ #ifdef __cplusplus extern "C" { #endif -LEAN_EXPORT uint64_t l___private_Lake_Build_Key_0__Lake_hashBuildKey____x40_Lake_Build_Key___hyg_1274_(lean_object*); lean_object* l_Lean_Name_reprPrec(lean_object*, lean_object*); -static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__6; -LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_hashBuildKey____x40_Lake_Build_Key___hyg_1274____boxed(lean_object*); +LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0____private_Lake_Build_Key_0__Lake_reprBuildKey_match__1_splitter____x40_Lake_Build_Key___hyg_93____rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_hashBuildKey____x40_Lake_Build_Key___hyg_1275____boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_BuildKey_quickCmp_match__1_splitter(lean_object*); -LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_325____boxed(lean_object*, lean_object*); +static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__2; +LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_326____boxed(lean_object*, lean_object*); +static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__9; uint64_t lean_uint64_mix_hash(uint64_t, uint64_t); +static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__13; lean_object* l_Lean_Name_toString(lean_object*, uint8_t, lean_object*); -LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0____private_Lake_Build_Key_0__Lake_reprBuildKey_match__1_splitter____x40_Lake_Build_Key___hyg_92____rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__8; -static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__9; -static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__14; -LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____boxed(lean_object*, lean_object*); -static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__12; -LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0____private_Lake_Build_Key_0__Lake_reprBuildKey_match__1_splitter____x40_Lake_Build_Key___hyg_92_(lean_object*); +static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__7; +LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0____private_Lake_Build_Key_0__Lake_reprBuildKey_match__1_splitter____x40_Lake_Build_Key___hyg_93_(lean_object*); +static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__8; +static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__14; LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_BuildKey_quickCmp_match__4_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__3; LEAN_EXPORT lean_object* l_Lake_BuildKey_quickCmp___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_BuildKey_quickCmp_match__5_splitter(lean_object*); +static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__12; static lean_object* l_Lake_instInhabitedBuildKey___closed__1; +LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_BuildKey_quickCmp_match__2_splitter(lean_object*); lean_object* lean_nat_to_int(lean_object*); +static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__3; LEAN_EXPORT lean_object* l_Lake_instReprBuildKey; -static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__1; LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_BuildKey_quickCmp_match__3_splitter(lean_object*); -LEAN_EXPORT uint8_t l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_325_(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____boxed(lean_object*, lean_object*); lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_BuildKey_toSimpleString(lean_object*); LEAN_EXPORT lean_object* l_Lake_BuildKey_toSimpleString_eraseHead(lean_object*); @@ -47,7 +47,10 @@ LEAN_EXPORT lean_object* l_Lake_BuildKey_toString(lean_object*); uint8_t lean_name_eq(lean_object*, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l_Lake_BuildKey_toString___closed__1; -LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92_(lean_object*, lean_object*); +LEAN_EXPORT uint64_t l___private_Lake_Build_Key_0__Lake_hashBuildKey____x40_Lake_Build_Key___hyg_1275_(lean_object*); +static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__5; +static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__6; +static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__1; LEAN_EXPORT uint8_t l_Lake_BuildKey_toString___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Lake_instInhabitedBuildKey; LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_BuildKey_quickCmp_match__5_splitter___rarg(lean_object*, lean_object*, lean_object*); @@ -55,31 +58,28 @@ LEAN_EXPORT lean_object* l_Lake_instHashableBuildKey; LEAN_EXPORT lean_object* l_Lake_instDecidableEqBuildKey___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_BuildKey_quickCmp_match__3_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_BuildKey_instToString(lean_object*); +static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__10; LEAN_EXPORT lean_object* l_Lake_BuildKey_toString___lambda__1___boxed(lean_object*); static lean_object* l_Lake_BuildKey_toString___closed__3; -static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__11; -static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__7; +static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__11; uint64_t l_Lean_Name_hash___override(lean_object*); +static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__4; lean_object* l_Repr_addAppParen(lean_object*, lean_object*); static lean_object* l_Lake_instReprBuildKey___closed__1; -static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__10; static lean_object* l_Lake_instHashableBuildKey___closed__1; uint8_t l_Lean_Name_quickCmp(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_BuildKey_quickCmp_match__1_splitter___rarg(uint8_t, lean_object*, lean_object*); -static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__4; static lean_object* l_Lake_BuildKey_toString___closed__6; lean_object* lean_string_append(lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lake_BuildKey_quickCmp(lean_object*, lean_object*); -static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__13; +LEAN_EXPORT uint8_t l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_326_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_BuildKey_quickCmp_match__4_splitter(lean_object*); LEAN_EXPORT uint8_t l_Lake_instDecidableEqBuildKey(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_BuildKey_quickCmp_match__2_splitter___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_BuildKey_toString___closed__4; -static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__5; static lean_object* l_Lake_BuildKey_toString___closed__5; static lean_object* l_Lake_BuildKey_toString___closed__2; -static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__2; static lean_object* _init_l_Lake_instInhabitedBuildKey___closed__1() { _start: { @@ -99,7 +99,7 @@ x_1 = l_Lake_instInhabitedBuildKey___closed__1; return x_1; } } -static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__1() { +static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__1() { _start: { lean_object* x_1; @@ -107,21 +107,21 @@ x_1 = lean_mk_string_unchecked("Lake.BuildKey.moduleFacet", 25, 25); return x_1; } } -static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__2() { +static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__1; +x_1 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__1; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__3() { +static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__2; +x_1 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__2; x_2 = lean_box(1); x_3 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -129,7 +129,7 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__4() { +static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__4() { _start: { lean_object* x_1; lean_object* x_2; @@ -138,7 +138,7 @@ x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__5() { +static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__5() { _start: { lean_object* x_1; lean_object* x_2; @@ -147,7 +147,7 @@ x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__6() { +static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__6() { _start: { lean_object* x_1; @@ -155,21 +155,21 @@ x_1 = lean_mk_string_unchecked("Lake.BuildKey.packageFacet", 26, 26); return x_1; } } -static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__7() { +static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__7() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__6; +x_1 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__6; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__8() { +static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__7; +x_1 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__7; x_2 = lean_box(1); x_3 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -177,7 +177,7 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__9() { +static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__9() { _start: { lean_object* x_1; @@ -185,21 +185,21 @@ x_1 = lean_mk_string_unchecked("Lake.BuildKey.targetFacet", 25, 25); return x_1; } } -static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__10() { +static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__10() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__9; +x_1 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__9; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__11() { +static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__10; +x_1 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__10; x_2 = lean_box(1); x_3 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -207,7 +207,7 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__12() { +static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__12() { _start: { lean_object* x_1; @@ -215,21 +215,21 @@ x_1 = lean_mk_string_unchecked("Lake.BuildKey.customTarget", 26, 26); return x_1; } } -static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__13() { +static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__13() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__12; +x_1 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__12; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__14() { +static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__13; +x_1 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__13; x_2 = lean_box(1); x_3 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -237,7 +237,7 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92_(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93_(lean_object* x_1, lean_object* x_2) { _start: { switch (lean_obj_tag(x_1)) { @@ -253,7 +253,7 @@ x_5 = lean_ctor_get(x_1, 1); x_6 = lean_unsigned_to_nat(1024u); x_7 = lean_nat_dec_le(x_6, x_2); x_8 = l_Lean_Name_reprPrec(x_4, x_6); -x_9 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__3; +x_9 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__3; lean_ctor_set_tag(x_1, 5); lean_ctor_set(x_1, 1, x_8); lean_ctor_set(x_1, 0, x_9); @@ -268,7 +268,7 @@ lean_ctor_set(x_13, 1, x_12); if (x_7 == 0) { lean_object* x_14; lean_object* x_15; uint8_t x_16; lean_object* x_17; lean_object* x_18; -x_14 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__4; +x_14 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__4; x_15 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_15, 0, x_14); lean_ctor_set(x_15, 1, x_13); @@ -282,7 +282,7 @@ return x_18; else { lean_object* x_19; lean_object* x_20; uint8_t x_21; lean_object* x_22; lean_object* x_23; -x_19 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__5; +x_19 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__5; x_20 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_20, 0, x_19); lean_ctor_set(x_20, 1, x_13); @@ -305,7 +305,7 @@ lean_dec(x_1); x_26 = lean_unsigned_to_nat(1024u); x_27 = lean_nat_dec_le(x_26, x_2); x_28 = l_Lean_Name_reprPrec(x_24, x_26); -x_29 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__3; +x_29 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__3; x_30 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_30, 0, x_29); lean_ctor_set(x_30, 1, x_28); @@ -320,7 +320,7 @@ lean_ctor_set(x_34, 1, x_33); if (x_27 == 0) { lean_object* x_35; lean_object* x_36; uint8_t x_37; lean_object* x_38; lean_object* x_39; -x_35 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__4; +x_35 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__4; x_36 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_36, 0, x_35); lean_ctor_set(x_36, 1, x_34); @@ -334,7 +334,7 @@ return x_39; else { lean_object* x_40; lean_object* x_41; uint8_t x_42; lean_object* x_43; lean_object* x_44; -x_40 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__5; +x_40 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__5; x_41 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_41, 0, x_40); lean_ctor_set(x_41, 1, x_34); @@ -359,7 +359,7 @@ x_47 = lean_ctor_get(x_1, 1); x_48 = lean_unsigned_to_nat(1024u); x_49 = lean_nat_dec_le(x_48, x_2); x_50 = l_Lean_Name_reprPrec(x_46, x_48); -x_51 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__8; +x_51 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__8; lean_ctor_set_tag(x_1, 5); lean_ctor_set(x_1, 1, x_50); lean_ctor_set(x_1, 0, x_51); @@ -374,7 +374,7 @@ lean_ctor_set(x_55, 1, x_54); if (x_49 == 0) { lean_object* x_56; lean_object* x_57; uint8_t x_58; lean_object* x_59; lean_object* x_60; -x_56 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__4; +x_56 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__4; x_57 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_57, 0, x_56); lean_ctor_set(x_57, 1, x_55); @@ -388,7 +388,7 @@ return x_60; else { lean_object* x_61; lean_object* x_62; uint8_t x_63; lean_object* x_64; lean_object* x_65; -x_61 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__5; +x_61 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__5; x_62 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_62, 0, x_61); lean_ctor_set(x_62, 1, x_55); @@ -411,7 +411,7 @@ lean_dec(x_1); x_68 = lean_unsigned_to_nat(1024u); x_69 = lean_nat_dec_le(x_68, x_2); x_70 = l_Lean_Name_reprPrec(x_66, x_68); -x_71 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__8; +x_71 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__8; x_72 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_72, 0, x_71); lean_ctor_set(x_72, 1, x_70); @@ -426,7 +426,7 @@ lean_ctor_set(x_76, 1, x_75); if (x_69 == 0) { lean_object* x_77; lean_object* x_78; uint8_t x_79; lean_object* x_80; lean_object* x_81; -x_77 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__4; +x_77 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__4; x_78 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_78, 0, x_77); lean_ctor_set(x_78, 1, x_76); @@ -440,7 +440,7 @@ return x_81; else { lean_object* x_82; lean_object* x_83; uint8_t x_84; lean_object* x_85; lean_object* x_86; -x_82 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__5; +x_82 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__5; x_83 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_83, 0, x_82); lean_ctor_set(x_83, 1, x_76); @@ -466,7 +466,7 @@ lean_dec(x_1); x_90 = lean_unsigned_to_nat(1024u); x_91 = lean_nat_dec_le(x_90, x_2); x_92 = l_Lean_Name_reprPrec(x_87, x_90); -x_93 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__11; +x_93 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__11; x_94 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_94, 0, x_93); lean_ctor_set(x_94, 1, x_92); @@ -488,7 +488,7 @@ lean_ctor_set(x_101, 1, x_100); if (x_91 == 0) { lean_object* x_102; lean_object* x_103; uint8_t x_104; lean_object* x_105; lean_object* x_106; -x_102 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__4; +x_102 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__4; x_103 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_103, 0, x_102); lean_ctor_set(x_103, 1, x_101); @@ -502,7 +502,7 @@ return x_106; else { lean_object* x_107; lean_object* x_108; uint8_t x_109; lean_object* x_110; lean_object* x_111; -x_107 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__5; +x_107 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__5; x_108 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_108, 0, x_107); lean_ctor_set(x_108, 1, x_101); @@ -526,7 +526,7 @@ x_114 = lean_ctor_get(x_1, 1); x_115 = lean_unsigned_to_nat(1024u); x_116 = lean_nat_dec_le(x_115, x_2); x_117 = l_Lean_Name_reprPrec(x_113, x_115); -x_118 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__14; +x_118 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__14; lean_ctor_set_tag(x_1, 5); lean_ctor_set(x_1, 1, x_117); lean_ctor_set(x_1, 0, x_118); @@ -541,7 +541,7 @@ lean_ctor_set(x_122, 1, x_121); if (x_116 == 0) { lean_object* x_123; lean_object* x_124; uint8_t x_125; lean_object* x_126; lean_object* x_127; -x_123 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__4; +x_123 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__4; x_124 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_124, 0, x_123); lean_ctor_set(x_124, 1, x_122); @@ -555,7 +555,7 @@ return x_127; else { lean_object* x_128; lean_object* x_129; uint8_t x_130; lean_object* x_131; lean_object* x_132; -x_128 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__5; +x_128 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__5; x_129 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_129, 0, x_128); lean_ctor_set(x_129, 1, x_122); @@ -578,7 +578,7 @@ lean_dec(x_1); x_135 = lean_unsigned_to_nat(1024u); x_136 = lean_nat_dec_le(x_135, x_2); x_137 = l_Lean_Name_reprPrec(x_133, x_135); -x_138 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__14; +x_138 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__14; x_139 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_139, 0, x_138); lean_ctor_set(x_139, 1, x_137); @@ -593,7 +593,7 @@ lean_ctor_set(x_143, 1, x_142); if (x_136 == 0) { lean_object* x_144; lean_object* x_145; uint8_t x_146; lean_object* x_147; lean_object* x_148; -x_144 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__4; +x_144 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__4; x_145 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_145, 0, x_144); lean_ctor_set(x_145, 1, x_143); @@ -607,7 +607,7 @@ return x_148; else { lean_object* x_149; lean_object* x_150; uint8_t x_151; lean_object* x_152; lean_object* x_153; -x_149 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__5; +x_149 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__5; x_150 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_150, 0, x_149); lean_ctor_set(x_150, 1, x_143); @@ -623,11 +623,11 @@ return x_153; } } } -LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92_(x_1, x_2); +x_3 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93_(x_1, x_2); lean_dec(x_2); return x_3; } @@ -636,7 +636,7 @@ static lean_object* _init_l_Lake_instReprBuildKey___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____boxed), 2, 0); return x_1; } } @@ -648,7 +648,7 @@ x_1 = l_Lake_instReprBuildKey___closed__1; return x_1; } } -LEAN_EXPORT uint8_t l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_325_(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_326_(lean_object* x_1, lean_object* x_2) { _start: { switch (lean_obj_tag(x_1)) { @@ -788,11 +788,11 @@ return x_38; } } } -LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_325____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_326____boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_325_(x_1, x_2); +x_3 = l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_326_(x_1, x_2); lean_dec(x_2); lean_dec(x_1); x_4 = lean_box(x_3); @@ -803,7 +803,7 @@ LEAN_EXPORT uint8_t l_Lake_instDecidableEqBuildKey(lean_object* x_1, lean_object _start: { uint8_t x_3; -x_3 = l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_325_(x_1, x_2); +x_3 = l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_326_(x_1, x_2); return x_3; } } @@ -818,7 +818,7 @@ x_4 = lean_box(x_3); return x_4; } } -LEAN_EXPORT uint64_t l___private_Lake_Build_Key_0__Lake_hashBuildKey____x40_Lake_Build_Key___hyg_1274_(lean_object* x_1) { +LEAN_EXPORT uint64_t l___private_Lake_Build_Key_0__Lake_hashBuildKey____x40_Lake_Build_Key___hyg_1275_(lean_object* x_1) { _start: { switch (lean_obj_tag(x_1)) { @@ -876,11 +876,11 @@ return x_32; } } } -LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_hashBuildKey____x40_Lake_Build_Key___hyg_1274____boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_hashBuildKey____x40_Lake_Build_Key___hyg_1275____boxed(lean_object* x_1) { _start: { uint64_t x_2; lean_object* x_3; -x_2 = l___private_Lake_Build_Key_0__Lake_hashBuildKey____x40_Lake_Build_Key___hyg_1274_(x_1); +x_2 = l___private_Lake_Build_Key_0__Lake_hashBuildKey____x40_Lake_Build_Key___hyg_1275_(x_1); lean_dec(x_1); x_3 = lean_box_uint64(x_2); return x_3; @@ -890,7 +890,7 @@ static lean_object* _init_l_Lake_instHashableBuildKey___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lake_Build_Key_0__Lake_hashBuildKey____x40_Lake_Build_Key___hyg_1274____boxed), 1, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lake_Build_Key_0__Lake_hashBuildKey____x40_Lake_Build_Key___hyg_1275____boxed), 1, 0); return x_1; } } @@ -1427,7 +1427,7 @@ lean_dec(x_2); return x_5; } } -LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0____private_Lake_Build_Key_0__Lake_reprBuildKey_match__1_splitter____x40_Lake_Build_Key___hyg_92____rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0____private_Lake_Build_Key_0__Lake_reprBuildKey_match__1_splitter____x40_Lake_Build_Key___hyg_93____rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { switch (lean_obj_tag(x_1)) { @@ -1492,11 +1492,11 @@ return x_18; } } } -LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0____private_Lake_Build_Key_0__Lake_reprBuildKey_match__1_splitter____x40_Lake_Build_Key___hyg_92_(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0____private_Lake_Build_Key_0__Lake_reprBuildKey_match__1_splitter____x40_Lake_Build_Key___hyg_93_(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l___private_Lake_Build_Key_0____private_Lake_Build_Key_0__Lake_reprBuildKey_match__1_splitter____x40_Lake_Build_Key___hyg_92____rarg), 5, 0); +x_2 = lean_alloc_closure((void*)(l___private_Lake_Build_Key_0____private_Lake_Build_Key_0__Lake_reprBuildKey_match__1_splitter____x40_Lake_Build_Key___hyg_93____rarg), 5, 0); return x_2; } } @@ -1681,34 +1681,34 @@ l_Lake_instInhabitedBuildKey___closed__1 = _init_l_Lake_instInhabitedBuildKey___ lean_mark_persistent(l_Lake_instInhabitedBuildKey___closed__1); l_Lake_instInhabitedBuildKey = _init_l_Lake_instInhabitedBuildKey(); lean_mark_persistent(l_Lake_instInhabitedBuildKey); -l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__1 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__1(); -lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__1); -l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__2 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__2(); -lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__2); -l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__3 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__3(); -lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__3); -l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__4 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__4(); -lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__4); -l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__5 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__5(); -lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__5); -l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__6 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__6(); -lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__6); -l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__7 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__7(); -lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__7); -l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__8 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__8(); -lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__8); -l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__9 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__9(); -lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__9); -l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__10 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__10(); -lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__10); -l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__11 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__11(); -lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__11); -l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__12 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__12(); -lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__12); -l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__13 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__13(); -lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__13); -l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__14 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__14(); -lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__14); +l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__1 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__1(); +lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__1); +l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__2 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__2(); +lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__2); +l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__3 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__3(); +lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__3); +l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__4 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__4(); +lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__4); +l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__5 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__5(); +lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__5); +l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__6 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__6(); +lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__6); +l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__7 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__7(); +lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__7); +l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__8 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__8(); +lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__8); +l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__9 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__9(); +lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__9); +l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__10 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__10(); +lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__10); +l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__11 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__11(); +lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__11); +l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__12 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__12(); +lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__12); +l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__13 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__13(); +lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__13); +l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__14 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__14(); +lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__14); l_Lake_instReprBuildKey___closed__1 = _init_l_Lake_instReprBuildKey___closed__1(); lean_mark_persistent(l_Lake_instReprBuildKey___closed__1); l_Lake_instReprBuildKey = _init_l_Lake_instReprBuildKey(); diff --git a/stage0/stdlib/Lake/Build/Module.c b/stage0/stdlib/Lake/Build/Module.c index 81c74e0176ad..7c30418300c8 100644 --- a/stage0/stdlib/Lake/Build/Module.c +++ b/stage0/stdlib/Lake/Build/Module.c @@ -20,6 +20,7 @@ static lean_object* l_Lake_Module_transImportsFacetConfig___closed__1; lean_object* l_Lake_compileO(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lake_Module_bcFile_x3f(lean_object*); static lean_object* l_Lake_Module_recBuildLeanCToOExport___closed__4; +lean_object* l_Array_take___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_OrdHashSet_insert___at_Lake_Module_recParseImports___spec__2(lean_object*, lean_object*); static lean_object* l_Lake_Module_dynlibFacetConfig___closed__2; static lean_object* l_Lake_Module_leanArtsFacetConfig___closed__3; @@ -330,7 +331,6 @@ lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); static lean_object* l_Lake_Module_depsFacetConfig___closed__3; LEAN_EXPORT lean_object* l_Lean_RBNode_fold___at_Lake_recBuildExternDynlibs___spec__1(lean_object*, lean_object*, lean_object*); lean_object* l_Lake_BuildJob_mixArray___rarg(lean_object*); -lean_object* l_Array_shrink___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_Module_recBuildDeps___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_parseImports_x27(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lake_Module_recBuildDynlib___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -4729,7 +4729,7 @@ if (x_118 == 0) lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_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; 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_119 = lean_ctor_get(x_111, 0); x_120 = lean_ctor_get(x_111, 1); -x_121 = l_Array_shrink___rarg(x_120, x_119); +x_121 = l_Array_take___rarg(x_120, x_119); lean_dec(x_119); x_122 = l_Array_forInUnsafe_loop___at_Lake_collectImportsAux___spec__3___closed__1; x_123 = lean_string_append(x_122, x_1); @@ -4777,7 +4777,7 @@ x_141 = lean_ctor_get(x_111, 1); lean_inc(x_141); lean_inc(x_140); lean_dec(x_111); -x_142 = l_Array_shrink___rarg(x_141, x_140); +x_142 = l_Array_take___rarg(x_141, x_140); lean_dec(x_140); x_143 = l_Array_forInUnsafe_loop___at_Lake_collectImportsAux___spec__3___closed__1; x_144 = lean_string_append(x_143, x_1); @@ -4837,7 +4837,7 @@ if (lean_is_exclusive(x_111)) { lean_dec_ref(x_111); x_165 = lean_box(0); } -x_166 = l_Array_shrink___rarg(x_164, x_163); +x_166 = l_Array_take___rarg(x_164, x_163); lean_dec(x_163); x_167 = l_Array_forInUnsafe_loop___at_Lake_collectImportsAux___spec__3___closed__1; x_168 = lean_string_append(x_167, x_1); @@ -6059,7 +6059,7 @@ if (x_117 == 0) lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; 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_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; x_118 = lean_ctor_get(x_110, 0); x_119 = lean_ctor_get(x_110, 1); -x_120 = l_Array_shrink___rarg(x_119, x_118); +x_120 = l_Array_take___rarg(x_119, x_118); lean_dec(x_118); x_121 = l_Array_forInUnsafe_loop___at_Lake_collectImportsAux___spec__3___closed__1; x_122 = lean_string_append(x_121, x_1); @@ -6107,7 +6107,7 @@ x_140 = lean_ctor_get(x_110, 1); lean_inc(x_140); lean_inc(x_139); lean_dec(x_110); -x_141 = l_Array_shrink___rarg(x_140, x_139); +x_141 = l_Array_take___rarg(x_140, x_139); lean_dec(x_139); x_142 = l_Array_forInUnsafe_loop___at_Lake_collectImportsAux___spec__3___closed__1; x_143 = lean_string_append(x_142, x_1); @@ -6167,7 +6167,7 @@ if (lean_is_exclusive(x_110)) { lean_dec_ref(x_110); x_164 = lean_box(0); } -x_165 = l_Array_shrink___rarg(x_163, x_162); +x_165 = l_Array_take___rarg(x_163, x_162); lean_dec(x_162); x_166 = l_Array_forInUnsafe_loop___at_Lake_collectImportsAux___spec__3___closed__1; x_167 = lean_string_append(x_166, x_1); @@ -8310,7 +8310,7 @@ if (x_117 == 0) lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; 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_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; x_118 = lean_ctor_get(x_110, 0); x_119 = lean_ctor_get(x_110, 1); -x_120 = l_Array_shrink___rarg(x_119, x_118); +x_120 = l_Array_take___rarg(x_119, x_118); lean_dec(x_118); x_121 = l_Array_forInUnsafe_loop___at_Lake_collectImportsAux___spec__3___closed__1; x_122 = lean_string_append(x_121, x_1); @@ -8358,7 +8358,7 @@ x_140 = lean_ctor_get(x_110, 1); lean_inc(x_140); lean_inc(x_139); lean_dec(x_110); -x_141 = l_Array_shrink___rarg(x_140, x_139); +x_141 = l_Array_take___rarg(x_140, x_139); lean_dec(x_139); x_142 = l_Array_forInUnsafe_loop___at_Lake_collectImportsAux___spec__3___closed__1; x_143 = lean_string_append(x_142, x_1); @@ -8418,7 +8418,7 @@ if (lean_is_exclusive(x_110)) { lean_dec_ref(x_110); x_164 = lean_box(0); } -x_165 = l_Array_shrink___rarg(x_163, x_162); +x_165 = l_Array_take___rarg(x_163, x_162); lean_dec(x_162); x_166 = l_Array_forInUnsafe_loop___at_Lake_collectImportsAux___spec__3___closed__1; x_167 = lean_string_append(x_166, x_1); @@ -10281,7 +10281,7 @@ if (x_117 == 0) lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; 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_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; x_118 = lean_ctor_get(x_110, 0); x_119 = lean_ctor_get(x_110, 1); -x_120 = l_Array_shrink___rarg(x_119, x_118); +x_120 = l_Array_take___rarg(x_119, x_118); lean_dec(x_118); x_121 = l_Array_forInUnsafe_loop___at_Lake_collectImportsAux___spec__3___closed__1; x_122 = lean_string_append(x_121, x_1); @@ -10329,7 +10329,7 @@ x_140 = lean_ctor_get(x_110, 1); lean_inc(x_140); lean_inc(x_139); lean_dec(x_110); -x_141 = l_Array_shrink___rarg(x_140, x_139); +x_141 = l_Array_take___rarg(x_140, x_139); lean_dec(x_139); x_142 = l_Array_forInUnsafe_loop___at_Lake_collectImportsAux___spec__3___closed__1; x_143 = lean_string_append(x_142, x_1); @@ -10389,7 +10389,7 @@ if (lean_is_exclusive(x_110)) { lean_dec_ref(x_110); x_164 = lean_box(0); } -x_165 = l_Array_shrink___rarg(x_163, x_162); +x_165 = l_Array_take___rarg(x_163, x_162); lean_dec(x_162); x_166 = l_Array_forInUnsafe_loop___at_Lake_collectImportsAux___spec__3___closed__1; x_167 = lean_string_append(x_166, x_1); diff --git a/stage0/stdlib/Lake/CLI/Init.c b/stage0/stdlib/Lake/CLI/Init.c index c970af835dda..7e2e9dd8da67 100644 --- a/stage0/stdlib/Lake/CLI/Init.c +++ b/stage0/stdlib/Lake/CLI/Init.c @@ -18,24 +18,24 @@ LEAN_EXPORT lean_object* l_Lake_defaultExeRoot; lean_object* lean_string_utf8_extract(lean_object*, lean_object*, lean_object*); lean_object* lean_format_pretty(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_mathToolchainUrl___closed__1; -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__7; lean_object* l_instBEqOfDecidableEq___rarg(lean_object*, lean_object*, lean_object*); uint32_t lean_string_utf8_get(lean_object*, lean_object*); static lean_object* l_Lake_stdLeanConfigFileContents___closed__3; LEAN_EXPORT lean_object* l_Lake_initPkg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_String_anyAux___at_Lake_validatePkgName___spec__2___closed__4___boxed__const__1; static lean_object* l_Lake_escapeName_x21___closed__1; -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__20; lean_object* lean_io_prim_handle_put_str(lean_object*, lean_object*, lean_object*); static lean_object* l_String_anyAux___at_Lake_validatePkgName___spec__2___closed__3; static lean_object* l_Lake_initPkg___lambda__2___closed__11; static lean_object* l_Lake_mainFileName___closed__3; LEAN_EXPORT lean_object* l_Lake_leanActionWorkflowContents; +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__5; LEAN_EXPORT lean_object* l_Lake_initPkg(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*); lean_object* l_System_FilePath_join(lean_object*, lean_object*); +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__1; LEAN_EXPORT lean_object* l_Lake_libRootFileContents(lean_object*, lean_object*); -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__1; LEAN_EXPORT lean_object* l_Lake_libRootFileContents___lambda__1___boxed(lean_object*); +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__10; LEAN_EXPORT lean_object* l_Lake_toolchainFileName; static lean_object* l_Lake_validatePkgName___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lake_createLeanActionWorkflow(lean_object*, lean_object*, lean_object*); @@ -43,14 +43,12 @@ static lean_object* l_Lake_mainFileContents___closed__2; static lean_object* l_Lake_defaultExeRoot___closed__1; static lean_object* l_Lake_escapeName_x21___closed__3; static lean_object* l_Lake_createLeanActionWorkflow___closed__7; -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__15; LEAN_EXPORT lean_object* l_Lake_InitTemplate_noConfusion___rarg___lambda__1(lean_object*); static lean_object* l_Lake_validatePkgName___lambda__1___closed__4; static lean_object* l_Lake_initPkg___lambda__2___closed__6; LEAN_EXPORT lean_object* l_Lake_validatePkgName___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_createLeanActionWorkflow___closed__4; lean_object* l_String_quote(lean_object*); -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__25; static lean_object* l_Lake_stdTomlConfigFileContents___closed__5; lean_object* l_Lean_Name_toString(lean_object*, uint8_t, lean_object*); LEAN_EXPORT uint8_t l_String_anyAux___at_Lake_validatePkgName___spec__2(lean_object*, lean_object*, lean_object*); @@ -59,9 +57,9 @@ uint8_t lean_nat_dec_le(lean_object*, lean_object*); static lean_object* l_Lake_initPkg___lambda__1___closed__4; lean_object* lean_array_push(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_InitTemplate_noConfusion(lean_object*); -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__11; static lean_object* l_Lake_stdTomlConfigFileContents___closed__4; static lean_object* l_Lake_gitignoreContents___closed__5; +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__8; static lean_object* l_Lake_createLeanActionWorkflow___lambda__1___closed__2; lean_object* l_instDecidableEqChar___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_escapeName_x21___boxed(lean_object*); @@ -71,69 +69,66 @@ static lean_object* l_Lake_mathToolchainBlobUrl___closed__1; lean_object* l_System_FilePath_withExtension(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lake_libRootFileContents___lambda__1(lean_object*); static lean_object* l_Lake_mainFileName___closed__4; -LEAN_EXPORT lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____boxed(lean_object*, lean_object*); static lean_object* l_Lake_initPkg___lambda__2___closed__4; LEAN_EXPORT lean_object* l_Lake_new___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_instReprInitTemplate; static lean_object* l_Lake_initPkg___lambda__6___closed__2; -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__4; -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__5; static lean_object* l_Lake_mathTomlConfigFileContents___closed__2; static lean_object* l_Lake_mathLeanConfigFileContents___closed__2; static lean_object* l_Lake_initPkg___lambda__1___closed__9; +LEAN_EXPORT lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415_(uint8_t, lean_object*); static lean_object* l_Lake_validatePkgName___lambda__1___closed__5; static lean_object* l_Lake_InitTemplate_ofString_x3f___closed__4; static lean_object* l_Lake_initPkg___lambda__1___closed__10; +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__26; +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__24; LEAN_EXPORT lean_object* l_Lake_InitTemplate_ofString_x3f___boxed(lean_object*); lean_object* lean_string_utf8_set(lean_object*, lean_object*, uint32_t); +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__25; extern uint32_t l_Lean_idBeginEscape; -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__8; -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__12; static lean_object* l_Lake_basicFileContents___closed__1; uint8_t lean_string_dec_eq(lean_object*, lean_object*); static lean_object* l_Lake_createLeanActionWorkflow___closed__5; +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__21; static lean_object* l_Lake_InitTemplate_ofString_x3f___closed__3; lean_object* l_System_FilePath_pathExists(lean_object*, lean_object*); static lean_object* l_Lake_libLeanConfigFileContents___closed__2; +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__23; lean_object* lean_string_utf8_byte_size(lean_object*); static lean_object* l_Lake_initPkg___lambda__2___closed__3; lean_object* lean_string_push(lean_object*, uint32_t); +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__3; +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__20; LEAN_EXPORT uint8_t l_Lake_instInhabitedInitTemplate; LEAN_EXPORT lean_object* l_Lake_mathToolchainUrl; lean_object* l_IO_FS_createDirAll(lean_object*, lean_object*); -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__9; LEAN_EXPORT lean_object* l_String_anyAux___at_Lake_validatePkgName___spec__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_mathTomlConfigFileContents___boxed(lean_object*, lean_object*); static lean_object* l_Lake_initPkg___lambda__2___closed__17; LEAN_EXPORT lean_object* l_Lake_initPkg___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_InitTemplate_ofString_x3f___closed__8; static lean_object* l_Lake_stdTomlConfigFileContents___closed__3; -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__6; static lean_object* l_Lake_toolchainFileName___closed__1; LEAN_EXPORT lean_object* l_Lake_initPkg___lambda__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_validatePkgName___lambda__1___closed__7; static lean_object* l_Lake_escapeName_x21___closed__4; static lean_object* l_Lake_exeTomlConfigFileContents___closed__1; -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__10; LEAN_EXPORT lean_object* l_Lake_initPkg___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_InitTemplate_configFileContents(uint8_t, uint8_t, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414_(uint8_t, lean_object*); lean_object* lean_string_utf8_next(lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_instDecidableEqInitTemplate___boxed(lean_object*, lean_object*); lean_object* l_System_FilePath_isDir(lean_object*, lean_object*); -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__21; LEAN_EXPORT lean_object* l_String_anyAux___at_Lake_validatePkgName___spec__2___closed__3___boxed__const__1; LEAN_EXPORT lean_object* l_Lake_gitignoreContents; -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__16; LEAN_EXPORT lean_object* l_Lake_escapeIdent___boxed(lean_object*); lean_object* lean_nat_to_int(lean_object*); static lean_object* l_Lake_validatePkgName___lambda__1___closed__3; static lean_object* l_Lake_initPkg___lambda__2___closed__14; -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__3; static lean_object* l_Lake_initPkg___lambda__2___closed__18; static lean_object* l_Lake_createLeanActionWorkflow___closed__3; static lean_object* l_Lake_instReprInitTemplate___closed__1; +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__22; static lean_object* l_Lake_validatePkgName___lambda__1___closed__10; LEAN_EXPORT lean_object* l_Lake_dotlessName(lean_object*); static lean_object* l_Lake_initPkg___lambda__2___closed__2; @@ -145,25 +140,26 @@ lean_object* l_Lake_stringToLegalOrSimpleName(lean_object*); LEAN_EXPORT lean_object* l_Lake_readmeFileContents___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lake_initPkg___lambda__1(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_initPkg___lambda__4(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__11; static lean_object* l_Lake_initPkg___closed__2; static lean_object* l_String_anyAux___at_Lake_validatePkgName___spec__2___closed__1; -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__19; static lean_object* l_Lake_initPkg___lambda__2___closed__10; LEAN_EXPORT lean_object* l_Lake_InitTemplate_ofNat___boxed(lean_object*); -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__14; lean_object* l_System_FilePath_fileName(lean_object*); static lean_object* l_Lake_gitignoreContents___closed__2; LEAN_EXPORT lean_object* l_Lake_mainFileName; static lean_object* l_Lake_InitTemplate_ofString_x3f___closed__5; static lean_object* l_String_anyAux___at_Lake_validatePkgName___spec__2___closed__2; +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__19; uint8_t lean_string_utf8_at_end(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_initPkg___lambda__6(lean_object*, lean_object*, uint8_t, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_panic___at_String_fromUTF8_x21___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lake_stdLeanConfigFileContents(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__4; lean_object* l_System_FilePath_addExtension(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_validatePkgName___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_initPkg___lambda__1___closed__6; -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__17; +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__2; static lean_object* l_Lake_createLeanActionWorkflow___closed__6; static lean_object* l_Lake_validatePkgName___closed__1; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); @@ -188,11 +184,14 @@ static lean_object* l_Lake_initPkg___closed__1; extern lean_object* l_Std_Format_defWidth; LEAN_EXPORT lean_object* l_Lake_basicFileContents; static lean_object* l_Lake_initPkg___lambda__1___closed__1; +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__14; static lean_object* l_Lake_initPkg___lambda__2___closed__8; static lean_object* l_Lake_stdLeanConfigFileContents___closed__1; static lean_object* l_Lake_stdTomlConfigFileContents___closed__1; static lean_object* l_Lake_escapeIdent___closed__2; +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__15; LEAN_EXPORT lean_object* l_Lake_initPkg___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__13; LEAN_EXPORT lean_object* l_Lake_createLeanActionWorkflow___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_mainFileName___closed__1; LEAN_EXPORT lean_object* l_Lake_init___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -227,26 +226,29 @@ static lean_object* l_Lake_validatePkgName___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Lake_exeFileContents; static lean_object* l_Lake_createLeanActionWorkflow___closed__2; LEAN_EXPORT lean_object* l_Lake_mathLeanConfigFileContents(lean_object*, lean_object*); +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__18; lean_object* lean_io_realpath(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_validatePkgName(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__6; static lean_object* l_Lake_initPkg___lambda__2___closed__9; LEAN_EXPORT lean_object* l_Lake_stdLeanConfigFileContents___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Repr_addAppParen(lean_object*, lean_object*); static lean_object* l_Lake_gitignoreContents___closed__1; +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__9; static lean_object* l_Lake_exeFileContents___closed__1; LEAN_EXPORT lean_object* l_Lake_libRootFileContents___boxed(lean_object*, lean_object*); static lean_object* l_Lake_validatePkgName___lambda__1___closed__6; +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__17; static lean_object* l_Lake_libRootFileContents___closed__3; LEAN_EXPORT lean_object* l_Lake_stdTomlConfigFileContents(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_mainFileContents(lean_object*); static lean_object* l_Lake_mathTomlConfigFileContents___closed__1; LEAN_EXPORT lean_object* l_Lake_InitTemplate_ofString_x3f(lean_object*); lean_object* l_Lake_proc(lean_object*, uint8_t, lean_object*, lean_object*); -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__22; +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__16; static lean_object* l_Lake_libRootFileContents___closed__1; LEAN_EXPORT lean_object* l_Lake_mathToolchainBlobUrl; LEAN_EXPORT lean_object* l_Lake_init(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__18; static lean_object* l_Lake_initPkg___lambda__2___closed__16; lean_object* l_Lake_toUpperCamelCase(lean_object*); lean_object* lean_array_mk(lean_object*); @@ -255,14 +257,12 @@ LEAN_EXPORT lean_object* l_String_mapAux___at_Lake_dotlessName___spec__1(lean_ob LEAN_EXPORT lean_object* l_Lake_escapeName_x21(lean_object*); LEAN_EXPORT lean_object* l_Lake_libLeanConfigFileContents(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_libTomlConfigFileContents(lean_object*, lean_object*); -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__13; lean_object* l_Lake_Env_toolchain(lean_object*); static lean_object* l_Lake_libRootFileContents___closed__2; static lean_object* l_Lake_mainFileName___closed__5; +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__12; LEAN_EXPORT lean_object* l_Lake_readmeFileContents(lean_object*); lean_object* lean_io_error_to_string(lean_object*); -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__26; -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__24; extern lean_object* l_Lake_defaultConfigFile; static lean_object* l_Lake_initPkg___lambda__2___closed__15; static lean_object* l_Lake_stdLeanConfigFileContents___closed__4; @@ -272,7 +272,6 @@ static lean_object* l_String_anyAux___at_Lake_validatePkgName___spec__2___closed lean_object* l_IO_FS_writeFile(lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_validatePkgName___lambda__1___closed__9; static lean_object* l_Lake_mainFileName___closed__2; -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__23; LEAN_EXPORT uint8_t l_Lake_instDecidableEqInitTemplate(uint8_t, uint8_t); lean_object* lean_string_append(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lake_InitTemplate_ofNat(lean_object*); @@ -285,7 +284,9 @@ static lean_object* l_Lake_libLeanConfigFileContents___closed__1; uint8_t lean_nat_dec_le(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_exeTomlConfigFileContents___boxed(lean_object*, lean_object*); static lean_object* l_Lake_createLeanActionWorkflow___lambda__1___closed__1; +LEAN_EXPORT lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____boxed(lean_object*, lean_object*); static lean_object* l_Lake_initPkg___lambda__1___closed__7; +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__7; static lean_object* l_Lake_init___closed__1; LEAN_EXPORT lean_object* l_Lake_initPkg___lambda__3(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_gitignoreContents___closed__4; @@ -298,7 +299,6 @@ lean_object* l_instDecidableEqString___boxed(lean_object*, lean_object*); static lean_object* l_Lake_leanActionWorkflowContents___closed__1; LEAN_EXPORT lean_object* l_Lake_InitTemplate_toCtorIdx(uint8_t); static lean_object* l_Lake_defaultExeRoot___closed__2; -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__2; extern lean_object* l_Lake_Git_upstreamBranch; LEAN_EXPORT lean_object* l_Lake_createLeanActionWorkflow___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* _init_l_Lake_defaultExeRoot___closed__1() { @@ -931,7 +931,7 @@ static lean_object* _init_l_Lake_mathLeanConfigFileContents___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked(" where\n version := v!\"0.1.0\"\n keywords := #[\"math\"]\n leanOptions := #[\n ⟨`pp.unicode.fun, true⟩ -- pretty-prints `fun a ↦ b`\n ]\n\nrequire \"leanprover-community\" / \"mathlib\"\n\n@[default_target]\nlean_lib ", 213, 207); +x_1 = lean_mk_string_unchecked(" where\n version := v!\"0.1.0\"\n keywords := #[\"math\"]\n leanOptions := #[\n ⟨`pp.unicode.fun, true⟩, -- pretty-prints `fun a ↦ b`\n ⟨`autoImplicit, false⟩\n ]\n\nrequire \"leanprover-community\" / \"mathlib\"\n\n@[default_target]\nlean_lib ", 245, 235); return x_1; } } @@ -986,7 +986,7 @@ static lean_object* _init_l_Lake_mathTomlConfigFileContents___closed__2() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("]\n\n[leanOptions]\npp.unicode.fun = true # pretty-prints `fun a ↦ b`\n\n[[require]]\nname = \"mathlib\"\nscope = \"leanprover-community\"\n\n[[lean_lib]]\nname = ", 151, 149); +x_1 = lean_mk_string_unchecked("]\n\n[leanOptions]\npp.unicode.fun = true # pretty-prints `fun a ↦ b`\nautoImplicit = false\n\n[[require]]\nname = \"mathlib\"\nscope = \"leanprover-community\"\n\n[[lean_lib]]\nname = ", 172, 170); return x_1; } } @@ -1198,7 +1198,7 @@ x_6 = l_Lake_InitTemplate_noConfusion___rarg(x_4, x_5, x_3); return x_6; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__1() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__1() { _start: { lean_object* x_1; @@ -1206,17 +1206,17 @@ x_1 = lean_mk_string_unchecked("Lake.InitTemplate.std", 21, 21); return x_1; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__2() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__1; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__1; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__3() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__3() { _start: { lean_object* x_1; lean_object* x_2; @@ -1225,23 +1225,23 @@ x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__4() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__3; -x_2 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__2; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__3; +x_2 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__2; x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__5() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__5() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__4; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__4; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -1249,7 +1249,7 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__6() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__6() { _start: { lean_object* x_1; lean_object* x_2; @@ -1258,23 +1258,23 @@ x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__7() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__6; -x_2 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__2; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__6; +x_2 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__2; x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__8() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__8() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__7; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__7; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -1282,7 +1282,7 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__9() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__9() { _start: { lean_object* x_1; @@ -1290,33 +1290,33 @@ x_1 = lean_mk_string_unchecked("Lake.InitTemplate.exe", 21, 21); return x_1; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__10() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__10() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__9; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__9; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__11() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__3; -x_2 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__10; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__3; +x_2 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__10; x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__12() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__12() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__11; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__11; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -1324,23 +1324,23 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__13() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__6; -x_2 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__10; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__6; +x_2 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__10; x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__14() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__14() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__13; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__13; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -1348,7 +1348,7 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__15() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__15() { _start: { lean_object* x_1; @@ -1356,33 +1356,33 @@ x_1 = lean_mk_string_unchecked("Lake.InitTemplate.lib", 21, 21); return x_1; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__16() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__16() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__15; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__15; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__17() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__17() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__3; -x_2 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__16; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__3; +x_2 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__16; x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__18() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__18() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__17; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__17; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -1390,23 +1390,23 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__19() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__19() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__6; -x_2 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__16; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__6; +x_2 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__16; x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__20() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__20() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__19; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__19; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -1414,7 +1414,7 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__21() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__21() { _start: { lean_object* x_1; @@ -1422,33 +1422,33 @@ x_1 = lean_mk_string_unchecked("Lake.InitTemplate.math", 22, 22); return x_1; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__22() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__22() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__21; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__21; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__23() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__23() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__3; -x_2 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__22; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__3; +x_2 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__22; x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__24() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__24() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__23; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__23; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -1456,23 +1456,23 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__25() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__25() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__6; -x_2 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__22; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__6; +x_2 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__22; x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__26() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__26() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__25; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__25; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -1480,7 +1480,7 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414_(uint8_t x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415_(uint8_t x_1, lean_object* x_2) { _start: { switch (x_1) { @@ -1492,14 +1492,14 @@ x_4 = lean_nat_dec_le(x_3, x_2); if (x_4 == 0) { lean_object* x_5; lean_object* x_6; -x_5 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__5; +x_5 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__5; x_6 = l_Repr_addAppParen(x_5, x_2); return x_6; } else { lean_object* x_7; lean_object* x_8; -x_7 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__8; +x_7 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__8; x_8 = l_Repr_addAppParen(x_7, x_2); return x_8; } @@ -1512,14 +1512,14 @@ x_10 = lean_nat_dec_le(x_9, x_2); if (x_10 == 0) { lean_object* x_11; lean_object* x_12; -x_11 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__12; +x_11 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__12; x_12 = l_Repr_addAppParen(x_11, x_2); return x_12; } else { lean_object* x_13; lean_object* x_14; -x_13 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__14; +x_13 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__14; x_14 = l_Repr_addAppParen(x_13, x_2); return x_14; } @@ -1532,14 +1532,14 @@ x_16 = lean_nat_dec_le(x_15, x_2); if (x_16 == 0) { lean_object* x_17; lean_object* x_18; -x_17 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__18; +x_17 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__18; x_18 = l_Repr_addAppParen(x_17, x_2); return x_18; } else { lean_object* x_19; lean_object* x_20; -x_19 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__20; +x_19 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__20; x_20 = l_Repr_addAppParen(x_19, x_2); return x_20; } @@ -1552,14 +1552,14 @@ x_22 = lean_nat_dec_le(x_21, x_2); if (x_22 == 0) { lean_object* x_23; lean_object* x_24; -x_23 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__24; +x_23 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__24; x_24 = l_Repr_addAppParen(x_23, x_2); return x_24; } else { lean_object* x_25; lean_object* x_26; -x_25 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__26; +x_25 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__26; x_26 = l_Repr_addAppParen(x_25, x_2); return x_26; } @@ -1567,13 +1567,13 @@ return x_26; } } } -LEAN_EXPORT lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; x_3 = lean_unbox(x_1); lean_dec(x_1); -x_4 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414_(x_3, x_2); +x_4 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415_(x_3, x_2); lean_dec(x_2); return x_4; } @@ -1582,7 +1582,7 @@ static lean_object* _init_l_Lake_instReprInitTemplate___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____boxed), 2, 0); return x_1; } } @@ -1891,7 +1891,7 @@ static lean_object* _init_l_Lake_escapeName_x21___closed__4() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lake_escapeName_x21___closed__1; x_2 = l_Lake_escapeName_x21___closed__2; -x_3 = lean_unsigned_to_nat(199u); +x_3 = lean_unsigned_to_nat(202u); x_4 = lean_unsigned_to_nat(23u); x_5 = l_Lake_escapeName_x21___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -1912,7 +1912,7 @@ static lean_object* _init_l_Lake_escapeName_x21___closed__6() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lake_escapeName_x21___closed__1; x_2 = l_Lake_escapeName_x21___closed__2; -x_3 = lean_unsigned_to_nat(202u); +x_3 = lean_unsigned_to_nat(205u); x_4 = lean_unsigned_to_nat(23u); x_5 = l_Lake_escapeName_x21___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -7002,58 +7002,58 @@ l_Lake_leanActionWorkflowContents = _init_l_Lake_leanActionWorkflowContents(); lean_mark_persistent(l_Lake_leanActionWorkflowContents); l_Lake_InitTemplate_noConfusion___rarg___closed__1 = _init_l_Lake_InitTemplate_noConfusion___rarg___closed__1(); lean_mark_persistent(l_Lake_InitTemplate_noConfusion___rarg___closed__1); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__1 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__1(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__1); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__2 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__2(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__2); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__3 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__3(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__3); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__4 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__4(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__4); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__5 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__5(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__5); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__6 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__6(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__6); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__7 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__7(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__7); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__8 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__8(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__8); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__9 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__9(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__9); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__10 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__10(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__10); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__11 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__11(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__11); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__12 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__12(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__12); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__13 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__13(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__13); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__14 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__14(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__14); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__15 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__15(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__15); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__16 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__16(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__16); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__17 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__17(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__17); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__18 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__18(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__18); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__19 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__19(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__19); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__20 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__20(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__20); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__21 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__21(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__21); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__22 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__22(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__22); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__23 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__23(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__23); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__24 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__24(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__24); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__25 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__25(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__25); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__26 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__26(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__26); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__1 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__1(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__1); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__2 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__2(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__2); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__3 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__3(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__3); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__4 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__4(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__4); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__5 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__5(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__5); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__6 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__6(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__6); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__7 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__7(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__7); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__8 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__8(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__8); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__9 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__9(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__9); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__10 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__10(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__10); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__11 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__11(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__11); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__12 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__12(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__12); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__13 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__13(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__13); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__14 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__14(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__14); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__15 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__15(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__15); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__16 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__16(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__16); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__17 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__17(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__17); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__18 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__18(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__18); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__19 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__19(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__19); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__20 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__20(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__20); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__21 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__21(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__21); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__22 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__22(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__22); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__23 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__23(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__23); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__24 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__24(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__24); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__25 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__25(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__25); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__26 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__26(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__26); l_Lake_instReprInitTemplate___closed__1 = _init_l_Lake_instReprInitTemplate___closed__1(); lean_mark_persistent(l_Lake_instReprInitTemplate___closed__1); l_Lake_instReprInitTemplate = _init_l_Lake_instReprInitTemplate(); diff --git a/stage0/stdlib/Lake/CLI/Main.c b/stage0/stdlib/Lake/CLI/Main.c index b8dd418d232b..0194e02b52d6 100644 --- a/stage0/stdlib/Lake/CLI/Main.c +++ b/stage0/stdlib/Lake/CLI/Main.c @@ -241,6 +241,7 @@ lean_object* l_Lake_loadWorkspace(lean_object*, uint8_t, lean_object*, lean_obje LEAN_EXPORT lean_object* l_Lake_lake_serve___lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_lake_checkBuild___lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_lake_resolveDeps___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); lean_object* lean_io_process_spawn(lean_object*, lean_object*); static lean_object* l_Lake_lakeCli___closed__5; static lean_object* l_Lake_lake_ReservoirConfig_currentSchemaVersion___closed__1; @@ -286,7 +287,6 @@ static lean_object* l_Lake_lakeCli___closed__2; LEAN_EXPORT lean_object* l_Lake_lake_test(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_lake_pack___lambda__2___boxed__const__1; LEAN_EXPORT lean_object* l_Lake_lake_versionTags(lean_object*, lean_object*, lean_object*); -lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); uint8_t l_Lake_BuildConfig_showProgress(lean_object*); static lean_object* l_Lake_lakeLongOption___closed__6; LEAN_EXPORT lean_object* l_Lake_lake_script_doc___lambda__1___boxed__const__1; @@ -55937,7 +55937,7 @@ x_81 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_81, 0, x_18); lean_ctor_set(x_81, 1, x_80); x_82 = l_Lake_CliStateM_runLogIO___rarg___closed__1; -x_83 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_81, x_82); +x_83 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_81, x_82); x_84 = l_Lean_Json_mkObj(x_83); return x_84; } @@ -55990,7 +55990,7 @@ x_100 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_100, 0, x_18); lean_ctor_set(x_100, 1, x_99); x_101 = l_Lake_CliStateM_runLogIO___rarg___closed__1; -x_102 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_100, x_101); +x_102 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_100, x_101); x_103 = l_Lean_Json_mkObj(x_102); return x_103; } @@ -56041,7 +56041,7 @@ x_119 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_119, 0, x_18); lean_ctor_set(x_119, 1, x_118); x_120 = l_Lake_CliStateM_runLogIO___rarg___closed__1; -x_121 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_119, x_120); +x_121 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_119, x_120); x_122 = l_Lean_Json_mkObj(x_121); return x_122; } diff --git a/stage0/stdlib/Lake/Config/Opaque.c b/stage0/stdlib/Lake/Config/Opaque.c index 348bedded3f9..97bd749741f3 100644 --- a/stage0/stdlib/Lake/Config/Opaque.c +++ b/stage0/stdlib/Lake/Config/Opaque.c @@ -13,10 +13,10 @@ #ifdef __cplusplus extern "C" { #endif -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_nonemptyType___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_nonemptyType___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_OpaquePackage_nonemptyType; LEAN_EXPORT lean_object* l_Lake_OpaqueWorkspace_nonemptyType; -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_nonemptyType(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_nonemptyType(lean_object*, lean_object*, lean_object*); static lean_object* _init_l_Lake_OpaquePackage_nonemptyType() { _start: { @@ -29,20 +29,20 @@ static lean_object* _init_l_Lake_OpaqueWorkspace_nonemptyType() { return lean_box(0); } } -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_nonemptyType(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_nonemptyType(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { return lean_box(0); } } -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_nonemptyType___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_nonemptyType___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_3; -x_3 = l_Lake_OpaqueTargetConfig_nonemptyType(x_1, x_2); +lean_object* x_4; +x_4 = l_Lake_OpaqueTargetConfig_nonemptyType(x_1, x_2, x_3); +lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -return x_3; +return x_4; } } lean_object* initialize_Init(uint8_t builtin, lean_object*); diff --git a/stage0/stdlib/Lake/Config/TargetConfig.c b/stage0/stdlib/Lake/Config/TargetConfig.c index 740ff3e6a224..623c20d43113 100644 --- a/stage0/stdlib/Lake/Config/TargetConfig.c +++ b/stage0/stdlib/Lake/Config/TargetConfig.c @@ -15,55 +15,55 @@ extern "C" { #endif LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_unsafeMk___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_RBNode_dFind___at_Lake_Package_findTargetConfig_x3f___spec__1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lake_OpaqueTargetConfig_instCoeTargetConfig__1___closed__1; +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instInhabitedNameOfTargetConfig(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instCoeNameTargetConfig___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_unsafeGet___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instInhabitedNameOfTargetConfig___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lake_mkTargetJobConfig(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instInhabitedOfTargetConfig___rarg___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_unsafeGet___rarg___boxed(lean_object*); -static lean_object* l_Lake_OpaqueTargetConfig_instCoeTargetConfig___closed__1; -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instInhabitedOfTargetConfig___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lake_Package_findTargetConfig_x3f___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instCoeTargetConfigName(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_unsafeMk___rarg___boxed(lean_object*); lean_object* lean_task_pure(lean_object*); LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_unsafeGet(lean_object*, lean_object*); static lean_object* l_Lake_instInhabitedTargetConfig___lambda__2___closed__5; LEAN_EXPORT lean_object* l_Lake_instInhabitedTargetConfig(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instInhabitedOfTargetConfig(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_unsafeMk___rarg(lean_object*); LEAN_EXPORT lean_object* l_Functor_discard___at_Lake_mkTargetJobConfig___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lake_instInhabitedTargetConfig___lambda__2___boxed(lean_object*); static lean_object* l_Functor_discard___at_Lake_mkTargetJobConfig___spec__1___rarg___closed__1; -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instInhabitedOfTargetConfig___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_instInhabitedTargetConfig___boxed(lean_object*, lean_object*); static lean_object* l_Lake_instInhabitedTargetConfig___closed__1; LEAN_EXPORT lean_object* l_Lake_Package_findTargetConfig_x3f(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instCoeTargetConfig___boxed(lean_object*, lean_object*); extern lean_object* l_Task_Priority_default; -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instCoeTargetConfig__1___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instCoeTargetConfig__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instCoeTargetConfigName___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_instInhabitedTargetConfig___lambda__2(lean_object*); static lean_object* l_Lake_instInhabitedTargetConfig___lambda__2___closed__4; extern lean_object* l_Lake_BuildTrace_nil; +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instInhabitedNameOfTargetConfig___rarg___boxed(lean_object*); lean_object* l_Lake_EResult_map___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_mkTargetJobConfig___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_RBNode_dFind___at_Lake_Package_findTargetConfig_x3f___spec__1___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lake_OpaqueTargetConfig_instCoeTargetConfigName___closed__1; LEAN_EXPORT lean_object* l_Lake_instInhabitedTargetConfig___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_instInhabitedTargetConfig___lambda__2___closed__3; static lean_object* l_Lake_instInhabitedTargetConfig___closed__2; static lean_object* l_Lake_instInhabitedTargetConfig___lambda__2___closed__6; static lean_object* l_Lake_instInhabitedTargetConfig___lambda__2___closed__7; LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_unsafeGet___rarg(lean_object*); -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instCoeTargetConfig(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instCoeNameTargetConfig(lean_object*, lean_object*); lean_object* lean_task_map(lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Functor_discard___at_Lake_mkTargetJobConfig___spec__1___rarg___lambda__1(lean_object*); static lean_object* l_Lake_instInhabitedTargetConfig___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_unsafeMk(lean_object*, lean_object*); lean_object* lean_array_mk(lean_object*); uint8_t l_Lean_Name_quickCmp(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instInhabitedNameOfTargetConfig___boxed(lean_object*, lean_object*); static lean_object* l_Functor_discard___at_Lake_mkTargetJobConfig___spec__1___rarg___closed__2; LEAN_EXPORT lean_object* l_Functor_discard___at_Lake_mkTargetJobConfig___spec__1___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lake_instInhabitedTargetConfig___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_instInhabitedTargetConfig___lambda__2___closed__2; +static lean_object* l_Lake_OpaqueTargetConfig_instCoeNameTargetConfig___closed__1; LEAN_EXPORT lean_object* l_Lake_instInhabitedTargetConfig___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { @@ -370,7 +370,7 @@ lean_dec(x_1); return x_3; } } -static lean_object* _init_l_Lake_OpaqueTargetConfig_instCoeTargetConfig___closed__1() { +static lean_object* _init_l_Lake_OpaqueTargetConfig_instCoeTargetConfigName___closed__1() { _start: { lean_object* x_1; @@ -378,19 +378,19 @@ x_1 = lean_alloc_closure((void*)(l_Lake_OpaqueTargetConfig_unsafeMk___rarg___box return x_1; } } -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instCoeTargetConfig(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instCoeTargetConfigName(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Lake_OpaqueTargetConfig_instCoeTargetConfig___closed__1; +x_3 = l_Lake_OpaqueTargetConfig_instCoeTargetConfigName___closed__1; return x_3; } } -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instCoeTargetConfig___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instCoeTargetConfigName___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Lake_OpaqueTargetConfig_instCoeTargetConfig(x_1, x_2); +x_3 = l_Lake_OpaqueTargetConfig_instCoeTargetConfigName(x_1, x_2); lean_dec(x_2); lean_dec(x_1); return x_3; @@ -430,7 +430,7 @@ lean_dec(x_1); return x_3; } } -static lean_object* _init_l_Lake_OpaqueTargetConfig_instCoeTargetConfig__1___closed__1() { +static lean_object* _init_l_Lake_OpaqueTargetConfig_instCoeNameTargetConfig___closed__1() { _start: { lean_object* x_1; @@ -438,53 +438,53 @@ x_1 = lean_alloc_closure((void*)(l_Lake_OpaqueTargetConfig_unsafeGet___rarg___bo return x_1; } } -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instCoeTargetConfig__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instCoeNameTargetConfig(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Lake_OpaqueTargetConfig_instCoeTargetConfig__1___closed__1; +x_3 = l_Lake_OpaqueTargetConfig_instCoeNameTargetConfig___closed__1; return x_3; } } -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instCoeTargetConfig__1___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instCoeNameTargetConfig___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Lake_OpaqueTargetConfig_instCoeTargetConfig__1(x_1, x_2); +x_3 = l_Lake_OpaqueTargetConfig_instCoeNameTargetConfig(x_1, x_2); lean_dec(x_2); lean_dec(x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instInhabitedOfTargetConfig___rarg(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instInhabitedNameOfTargetConfig___rarg(lean_object* x_1) { _start: { lean_inc(x_1); return x_1; } } -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instInhabitedOfTargetConfig(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instInhabitedNameOfTargetConfig(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Lake_OpaqueTargetConfig_instInhabitedOfTargetConfig___rarg___boxed), 1, 0); +x_3 = lean_alloc_closure((void*)(l_Lake_OpaqueTargetConfig_instInhabitedNameOfTargetConfig___rarg___boxed), 1, 0); return x_3; } } -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instInhabitedOfTargetConfig___rarg___boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instInhabitedNameOfTargetConfig___rarg___boxed(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l_Lake_OpaqueTargetConfig_instInhabitedOfTargetConfig___rarg(x_1); +x_2 = l_Lake_OpaqueTargetConfig_instInhabitedNameOfTargetConfig___rarg(x_1); lean_dec(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instInhabitedOfTargetConfig___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instInhabitedNameOfTargetConfig___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Lake_OpaqueTargetConfig_instInhabitedOfTargetConfig(x_1, x_2); +x_3 = l_Lake_OpaqueTargetConfig_instInhabitedNameOfTargetConfig(x_1, x_2); lean_dec(x_2); lean_dec(x_1); return x_3; @@ -619,10 +619,10 @@ l_Functor_discard___at_Lake_mkTargetJobConfig___spec__1___rarg___closed__1 = _in lean_mark_persistent(l_Functor_discard___at_Lake_mkTargetJobConfig___spec__1___rarg___closed__1); l_Functor_discard___at_Lake_mkTargetJobConfig___spec__1___rarg___closed__2 = _init_l_Functor_discard___at_Lake_mkTargetJobConfig___spec__1___rarg___closed__2(); lean_mark_persistent(l_Functor_discard___at_Lake_mkTargetJobConfig___spec__1___rarg___closed__2); -l_Lake_OpaqueTargetConfig_instCoeTargetConfig___closed__1 = _init_l_Lake_OpaqueTargetConfig_instCoeTargetConfig___closed__1(); -lean_mark_persistent(l_Lake_OpaqueTargetConfig_instCoeTargetConfig___closed__1); -l_Lake_OpaqueTargetConfig_instCoeTargetConfig__1___closed__1 = _init_l_Lake_OpaqueTargetConfig_instCoeTargetConfig__1___closed__1(); -lean_mark_persistent(l_Lake_OpaqueTargetConfig_instCoeTargetConfig__1___closed__1); +l_Lake_OpaqueTargetConfig_instCoeTargetConfigName___closed__1 = _init_l_Lake_OpaqueTargetConfig_instCoeTargetConfigName___closed__1(); +lean_mark_persistent(l_Lake_OpaqueTargetConfig_instCoeTargetConfigName___closed__1); +l_Lake_OpaqueTargetConfig_instCoeNameTargetConfig___closed__1 = _init_l_Lake_OpaqueTargetConfig_instCoeNameTargetConfig___closed__1(); +lean_mark_persistent(l_Lake_OpaqueTargetConfig_instCoeNameTargetConfig___closed__1); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Lake/DSL/DeclUtil.c b/stage0/stdlib/Lake/DSL/DeclUtil.c index 88839bc2e1dc..dfedceb6da43 100644 --- a/stage0/stdlib/Lake/DSL/DeclUtil.c +++ b/stage0/stdlib/Lake/DSL/DeclUtil.c @@ -15,38 +15,41 @@ extern "C" { #endif lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); static lean_object* l_Lake_DSL_declField___closed__8; +LEAN_EXPORT lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__14(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__5___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__7; LEAN_EXPORT lean_object* l_Lake_DSL_simpleDeclSig; +LEAN_EXPORT lean_object* l_Array_sequenceMap___at_Lake_DSL_elabConfigDecl___spec__11(lean_object*, lean_object*); static lean_object* l_Lake_DSL_declValWhere___closed__7; static lean_object* l_Lake_DSL_bracketedSimpleBinder___closed__13; lean_object* l_Lean_Elab_addCompletionInfo___at_Lean_withSetOptionIn___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_DSL_elabConfigDecl___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); static lean_object* l_Lake_DSL_declValWhere___closed__10; +static lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__13; static lean_object* l_Lake_DSL_elabConfigDecl___lambda__1___closed__2; static lean_object* l_Lake_DSL_simpleBinder___closed__1; LEAN_EXPORT lean_object* l_Lake_DSL_declValStruct; static lean_object* l_Lake_DSL_elabConfigDecl___lambda__2___closed__2; static lean_object* l_Lake_DSL_elabConfigDecl___lambda__2___closed__23; -LEAN_EXPORT lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DSL_simpleDeclSig___closed__8; static lean_object* l_Lake_DSL_declValDo___closed__8; -static lean_object* l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__6___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__6(lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DSL_structDeclSig___closed__6; static lean_object* l_Lake_DSL_identOrStr___closed__9; +LEAN_EXPORT lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__3; LEAN_EXPORT lean_object* l_Lake_DSL_elabConfigDecl___lambda__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DSL_expandAttrs___closed__6; -static lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__5; LEAN_EXPORT lean_object* l_Lake_DSL_elabConfigDecl___lambda__8(lean_object*, 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*); static lean_object* l_Lake_DSL_identOrStr___closed__1; -LEAN_EXPORT lean_object* l_Array_sequenceMap_loop___at_Lake_DSL_elabConfigDecl___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_mkIdentFromRef___at_Lake_DSL_elabConfigDecl___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DSL_simpleBinder___closed__4; +static lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__1; lean_object* l_Lean_TSyntax_getString(lean_object*); static lean_object* l_Lake_DSL_bracketedSimpleBinder___closed__12; -LEAN_EXPORT lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__14; +LEAN_EXPORT lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__1; lean_object* l_Lean_Syntax_getId(lean_object*); static lean_object* l_Lake_DSL_identOrStr___closed__3; lean_object* lean_array_push(lean_object*, lean_object*); @@ -60,7 +63,6 @@ static lean_object* l_Lake_DSL_declValStruct___closed__2; LEAN_EXPORT lean_object* l_Lake_DSL_simpleBinder; static lean_object* l_Lake_DSL_elabConfigDecl___lambda__2___closed__1; static lean_object* l_Lake_DSL_structDeclSig___closed__7; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__4(size_t, size_t, lean_object*); lean_object* l_Lean_Syntax_getArgs(lean_object*); lean_object* l_Lean_replaceRef(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_DSL_elabConfigDecl___lambda__7(lean_object*, lean_object*); @@ -68,30 +70,30 @@ lean_object* l_Lean_Elab_Command_elabCommand(lean_object*, lean_object*, lean_ob lean_object* lean_array_fget(lean_object*, lean_object*); static lean_object* l_Lake_DSL_structDeclSig___closed__2; static lean_object* l_Lake_DSL_declValDo___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshIdent___at_Lake_DSL_elabConfigDecl___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DSL_identOrStr___closed__5; static lean_object* l_Lake_DSL_elabConfigDecl___lambda__2___closed__21; lean_object* l_Lean_Syntax_TSepArray_getElems___rarg(lean_object*); static lean_object* l_Lake_DSL_expandAttrs___closed__3; -static lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__4; static lean_object* l_Lake_DSL_structVal___closed__4; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__12(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_DSL_expandOptSimpleBinder___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_DSL_identOrStr; lean_object* l_Lean_logAt___at_Lean_Elab_Command_runLinters___spec__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DSL_simpleDeclSig___closed__9; -static lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__8; lean_object* l_Lean_mkIdentFrom(lean_object*, lean_object*, uint8_t); static lean_object* l_Lake_DSL_elabConfigDecl___lambda__3___closed__1; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DSL_structVal___closed__2; static lean_object* l_Lake_DSL_expandAttrs___closed__5; lean_object* l_Lean_Syntax_node5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__4; static lean_object* l_Lake_DSL_declField___closed__11; uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); static lean_object* l_Lake_DSL_declValDo___closed__12; static lean_object* l_Lake_DSL_expandAttrs___closed__1; lean_object* l_Lean_stringToMessageData(lean_object*); static lean_object* l_Lake_DSL_structVal___closed__7; +LEAN_EXPORT lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_sequenceMap_loop___at_Lake_DSL_elabConfigDecl___spec__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DSL_structVal___closed__16; LEAN_EXPORT lean_object* l_Lake_DSL_elabConfigDecl___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_Lake_DSL_declValStruct___closed__5; @@ -101,15 +103,16 @@ static lean_object* l_Lake_DSL_elabConfigDecl___lambda__2___closed__5; static lean_object* l_Lake_DSL_bracketedSimpleBinder___closed__9; LEAN_EXPORT lean_object* l_Lake_DSL_expandOptSimpleBinder___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_DSL_expandOptSimpleBinder___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lake_DSL_elabConfigDecl___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DSL_structVal___closed__11; static lean_object* l_Lake_DSL_simpleDeclSig___closed__4; static lean_object* l_Lake_DSL_expandAttrs___closed__2; lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshIdent___at_Lake_DSL_elabConfigDecl___spec__5(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DSL_declField___closed__4; +static lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; LEAN_EXPORT lean_object* l_Lake_DSL_bracketedSimpleBinder; static lean_object* l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__4; -static lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__13; LEAN_EXPORT lean_object* l_Lake_DSL_elabConfigDecl___lambda__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_DSL_declValWhere; static lean_object* l_Lake_DSL_identOrStr___closed__8; @@ -119,71 +122,76 @@ static lean_object* l_Lake_DSL_simpleDeclSig___closed__10; static lean_object* l_Lake_DSL_elabConfigDecl___lambda__2___closed__24; static lean_object* l_Lake_DSL_structVal___closed__6; static lean_object* l_Lake_DSL_structVal___closed__13; +LEAN_EXPORT lean_object* l_Lean_mkIdentFromRef___at_Lake_DSL_elabConfigDecl___spec__8(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DSL_elabConfigDecl___lambda__2___closed__22; static lean_object* l_Lake_DSL_declValWhere___closed__4; LEAN_EXPORT lean_object* l_Lake_DSL_elabConfigDecl___lambda__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_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__6___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_SourceInfo_fromRef(lean_object*, uint8_t); lean_object* l_Lean_Syntax_node6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_mkIdentFromRef___at_Lake_DSL_elabConfigDecl___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__10; +static lean_object* l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__7___closed__2; static lean_object* l_Lake_DSL_elabConfigDecl___lambda__2___closed__18; +static lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__2; static lean_object* l_Lake_DSL_identOrStr___closed__13; lean_object* l_Lean_Elab_Command_getRef(lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DSL_identOrStr___closed__12; -LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshIdent___at_Lake_DSL_elabConfigDecl___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DSL_identOrStr___closed__6; static lean_object* l_Lake_DSL_structVal___closed__18; lean_object* l_Lean_mkCIdentFrom(lean_object*, lean_object*, uint8_t); +lean_object* l_Lean_Elab_getBetterRef(lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__7; static lean_object* l_Lake_DSL_simpleBinder___closed__2; LEAN_EXPORT lean_object* l_Lake_DSL_elabConfigDecl___lambda__7___boxed(lean_object*, lean_object*); static lean_object* l_Lake_DSL_structVal___closed__21; lean_object* lean_st_ref_get(lean_object*, lean_object*); +static lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__4; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__5(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lake_DSL_structDeclSig; LEAN_EXPORT lean_object* l_Lake_DSL_elabConfigDecl___lambda__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__13(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__7___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DSL_structVal___closed__17; static lean_object* l_Lake_DSL_declField___closed__7; +static lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__9; static lean_object* l_Lake_DSL_declValWhere___closed__9; lean_object* l_Lean_Syntax_node3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DSL_declValWhere___closed__6; static lean_object* l_Lake_DSL_elabConfigDecl___lambda__2___closed__13; static lean_object* l_Lake_DSL_simpleBinder___closed__3; +static lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__8; LEAN_EXPORT lean_object* l_Lake_DSL_elabConfigDecl___lambda__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_sequenceMap___at_Lake_DSL_elabConfigDecl___spec__11___boxed(lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__11; lean_object* l_Lean_RBNode_insert___at_Lean_NameMap_insert___spec__1___rarg(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Command_getCurrMacroScope(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_DSL_elabConfigDecl___lambda__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DSL_simpleDeclSig___closed__3; static lean_object* l_Lake_DSL_declValDo___closed__14; lean_object* l_Lean_addMacroScope(lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__11; +static lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__2; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l_Lake_DSL_elabConfigDecl___lambda__2___closed__8; static lean_object* l_Lake_DSL_simpleDeclSig___closed__11; -static lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__2; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_node2(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__6; +static lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__12; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, 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*); lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); static lean_object* l_Lake_DSL_elabConfigDecl___lambda__2___closed__4; static lean_object* l_Lake_DSL_identOrStr___closed__11; static lean_object* l_Lake_DSL_declValDo___closed__1; uint8_t l_Lean_Syntax_matchesNull(lean_object*, lean_object*); static lean_object* l_Lake_DSL_elabConfigDecl___lambda__2___closed__20; -LEAN_EXPORT lean_object* l_Array_sequenceMap___at_Lake_DSL_elabConfigDecl___spec__10___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DSL_structDeclSig___closed__4; static lean_object* l_Lake_DSL_structVal___closed__9; -static lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__2; +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lake_DSL_elabConfigDecl___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DSL_declValDo___closed__15; static lean_object* l_Lake_DSL_declValDo___closed__4; LEAN_EXPORT lean_object* l_Lake_DSL_expandIdentOrStrAsIdent(lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__12; LEAN_EXPORT lean_object* l_Lake_DSL_structVal; static lean_object* l_Lake_DSL_structDeclSig___closed__9; static lean_object* l_Lake_DSL_structVal___closed__10; -static lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__1; static lean_object* l_Lake_DSL_structVal___closed__8; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__12___boxed(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_Lake_DSL_declValDo; lean_object* l_Lean_MessageData_ofExpr(lean_object*); @@ -193,22 +201,20 @@ static lean_object* l_Lake_DSL_declValWhere___closed__8; static lean_object* l_Lake_DSL_elabConfigDecl___lambda__2___closed__15; static lean_object* l_Lake_DSL_declField___closed__12; static lean_object* l_Lake_DSL_bracketedSimpleBinder___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__6___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DSL_structDeclSig___closed__1; lean_object* l_Lean_Syntax_node4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DSL_simpleDeclSig___closed__7; static lean_object* l_Lake_DSL_bracketedSimpleBinder___closed__7; lean_object* l_Lean_Elab_Command_withFreshMacroScope___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DSL_bracketedSimpleBinder___closed__4; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DSL_simpleDeclSig___closed__6; static lean_object* l_Lake_DSL_declField___closed__5; LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lake_DSL_elabConfigDecl___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DSL_declValDo___closed__6; -LEAN_EXPORT lean_object* l_Array_sequenceMap___at_Lake_DSL_elabConfigDecl___spec__10(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lake_DSL_elabConfigDecl___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__6; static lean_object* l_Lake_DSL_identOrStr___closed__14; -LEAN_EXPORT lean_object* l_Lean_mkIdentFromRef___at_Lake_DSL_elabConfigDecl___spec__7(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DSL_declValDo___closed__9; static lean_object* l_Lake_DSL_simpleDeclSig___closed__12; uint8_t lean_nat_dec_eq(lean_object*, lean_object*); @@ -229,55 +235,55 @@ static lean_object* l_Lake_DSL_elabConfigDecl___lambda__2___closed__6; static lean_object* l_Lake_DSL_structVal___closed__5; lean_object* l_Lean_Syntax_node1(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkSepArray(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__7(lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_isNone(lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__1; -LEAN_EXPORT lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DSL_declValWhere___closed__1; lean_object* lean_nat_sub(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__7___closed__1; static lean_object* l_Lake_DSL_bracketedSimpleBinder___closed__1; lean_object* l_Array_mkArray1___rarg(lean_object*); static lean_object* l_Lake_DSL_elabConfigDecl___lambda__2___closed__11; -static lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__5; static lean_object* l_Lake_DSL_declValStruct___closed__3; lean_object* l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__9; -LEAN_EXPORT lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___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_throwErrorAt___at_Lean_Elab_Command_elabSyntax___spec__14(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__18(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DSL_declValWhere___closed__3; static lean_object* l_Lake_DSL_structVal___closed__15; static lean_object* l_Lake_DSL_declValDo___closed__7; static lean_object* l_Lake_DSL_simpleDeclSig___closed__5; static lean_object* l_Lake_DSL_declValWhere___closed__2; static lean_object* l_Lake_DSL_identOrStr___closed__7; +LEAN_EXPORT lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshIdent___at_Lake_DSL_elabConfigDecl___spec__6(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); lean_object* lean_array_mk(lean_object*); static lean_object* l_Lake_DSL_declField___closed__1; static lean_object* l_Lake_DSL_expandAttrs___closed__4; +static lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__5; LEAN_EXPORT lean_object* l_Lake_DSL_elabConfigDecl___lambda__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); static lean_object* l_Lake_DSL_structVal___closed__14; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___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_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__5; -LEAN_EXPORT lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DSL_bracketedSimpleBinder___closed__10; LEAN_EXPORT lean_object* l_Lake_DSL_elabConfigDecl___lambda__6(lean_object*, lean_object*); static lean_object* l_Lake_DSL_identOrStr___closed__4; +static lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__14; static lean_object* l_Lake_DSL_elabConfigDecl___lambda__2___closed__9; -static lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; static lean_object* l_Lake_DSL_declField___closed__6; lean_object* lean_array_uget(lean_object*, size_t); static lean_object* l_Lake_DSL_declValDo___closed__5; size_t lean_array_size(lean_object*); static lean_object* l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__7___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DSL_elabConfigDecl___lambda__2___closed__7; static lean_object* l_Lake_DSL_bracketedSimpleBinder___closed__8; static lean_object* l_Lake_DSL_declValDo___closed__11; static lean_object* l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__1; static lean_object* l_Lake_DSL_declField___closed__3; static lean_object* l_Lake_DSL_bracketedSimpleBinder___closed__11; +static lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; static lean_object* l_Lake_DSL_declField___closed__2; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__4___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DSL_structVal___closed__1; lean_object* lean_array_get_size(lean_object*); static lean_object* l_Lake_DSL_elabConfigDecl___lambda__2___closed__14; @@ -291,7 +297,6 @@ static lean_object* l_Lake_DSL_bracketedSimpleBinder___closed__3; static lean_object* l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__3; lean_object* lean_nat_add(lean_object*, lean_object*); static lean_object* l_Lake_DSL_declValWhere___closed__5; -static lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__3; static lean_object* l_Lake_DSL_elabConfigDecl___lambda__2___closed__3; LEAN_EXPORT lean_object* l_Lake_DSL_elabConfigDecl___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DSL_structDeclSig___closed__3; @@ -301,7 +306,8 @@ static lean_object* l_Lake_DSL_bracketedSimpleBinder___closed__6; static lean_object* l_Lake_DSL_structVal___closed__3; static lean_object* l_Lake_DSL_structDeclSig___closed__5; LEAN_EXPORT lean_object* l_Lake_DSL_elabConfigDecl___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__5; +static lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__10; LEAN_EXPORT lean_object* l_Lake_DSL_elabConfigDecl___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DSL_bracketedSimpleBinder___closed__5; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); @@ -309,18 +315,16 @@ LEAN_EXPORT lean_object* l_Lake_DSL_elabConfigDecl___lambda__5___boxed(lean_obje lean_object* l_Lean_MessageData_ofName(lean_object*); static lean_object* l_Lake_DSL_declValStruct___closed__4; LEAN_EXPORT lean_object* l_Lake_DSL_elabConfigDecl___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__4; LEAN_EXPORT lean_object* l_Lake_DSL_elabConfigDecl___lambda__6___boxed(lean_object*, lean_object*); static lean_object* l_Lake_DSL_declValDo___closed__13; -LEAN_EXPORT lean_object* l_Array_sequenceMap_loop___at_Lake_DSL_elabConfigDecl___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lake_Name_quoteFrom(lean_object*, lean_object*); static lean_object* l_Lake_DSL_identOrStr___closed__10; static lean_object* l_Lake_DSL_structVal___closed__19; static lean_object* l_Lake_DSL_elabConfigDecl___lambda__2___closed__19; -static lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__3; -static lean_object* l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__6___closed__2; static lean_object* l_Lake_DSL_bracketedSimpleBinder___closed__14; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__7; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_sequenceMap_loop___at_Lake_DSL_elabConfigDecl___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* _init_l_Lake_DSL_expandAttrs___closed__1() { _start: { @@ -2248,6 +2252,94 @@ lean_dec(x_2); return x_4; } } +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lake_DSL_elabConfigDecl___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; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_5 = l_Lean_Elab_Command_getRef(x_2, x_3, x_4); +x_6 = lean_ctor_get(x_5, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_5, 1); +lean_inc(x_7); +lean_dec(x_5); +x_8 = lean_ctor_get(x_2, 4); +lean_inc(x_8); +lean_inc(x_8); +x_9 = l_Lean_Elab_getBetterRef(x_6, x_8); +lean_dec(x_6); +x_10 = l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1(x_1, x_2, x_3, x_7); +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_12 = lean_ctor_get(x_10, 0); +x_13 = lean_ctor_get(x_10, 1); +x_14 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_12, x_8, x_2, x_3, x_13); +lean_dec(x_2); +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 0) +{ +lean_object* x_16; +x_16 = lean_ctor_get(x_14, 0); +lean_ctor_set(x_10, 1, x_16); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set_tag(x_14, 1); +lean_ctor_set(x_14, 0, x_10); +return x_14; +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_14, 0); +x_18 = lean_ctor_get(x_14, 1); +lean_inc(x_18); +lean_inc(x_17); +lean_dec(x_14); +lean_ctor_set(x_10, 1, x_17); +lean_ctor_set(x_10, 0, x_9); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_10); +lean_ctor_set(x_19, 1, 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; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_20 = lean_ctor_get(x_10, 0); +x_21 = lean_ctor_get(x_10, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_10); +x_22 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_20, x_8, x_2, x_3, x_21); +lean_dec(x_2); +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +if (lean_is_exclusive(x_22)) { + lean_ctor_release(x_22, 0); + lean_ctor_release(x_22, 1); + x_25 = x_22; +} else { + lean_dec_ref(x_22); + x_25 = lean_box(0); +} +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_9); +lean_ctor_set(x_26, 1, x_23); +if (lean_is_scalar(x_25)) { + x_27 = lean_alloc_ctor(1, 2, 0); +} else { + x_27 = x_25; + lean_ctor_set_tag(x_27, 1); +} +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_24); +return x_27; +} +} +} LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lake_DSL_elabConfigDecl___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { @@ -2267,7 +2359,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_expandDeclId___spec__18(x_2, x_3, x_4, x_8); +x_12 = l_Lean_throwError___at_Lake_DSL_elabConfigDecl___spec__2(x_2, x_3, x_4, x_8); return x_12; } else @@ -2305,12 +2397,12 @@ lean_ctor_set(x_23, 7, x_19); lean_ctor_set(x_23, 8, x_20); lean_ctor_set(x_23, 9, x_21); lean_ctor_set_uint8(x_23, sizeof(void*)*10, x_22); -x_24 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__18(x_2, x_23, x_4, x_8); +x_24 = l_Lean_throwError___at_Lake_DSL_elabConfigDecl___spec__2(x_2, x_23, x_4, x_8); return x_24; } } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__1() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__1() { _start: { lean_object* x_1; @@ -2318,16 +2410,16 @@ x_1 = lean_mk_string_unchecked("ill-formed field declaration syntax", 35, 35); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__2() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__1; +x_1 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__3() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__3() { _start: { lean_object* x_1; @@ -2335,17 +2427,17 @@ x_1 = l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_box(0), lean_box(0)); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__4() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__3; +x_1 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___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_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__5() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__5() { _start: { lean_object* x_1; lean_object* x_2; @@ -2354,23 +2446,23 @@ x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__6() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__6() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__5; +x_1 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___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_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__7() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__7() { _start: { size_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = 5; -x_2 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__6; -x_3 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__5; +x_2 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_3 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__5; x_4 = lean_unsigned_to_nat(0u); x_5 = lean_alloc_ctor(0, 4, sizeof(size_t)*1); lean_ctor_set(x_5, 0, x_2); @@ -2381,19 +2473,19 @@ lean_ctor_set_usize(x_5, 4, x_1); return x_5; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__8() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__4; -x_2 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__7; +x_1 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__4; +x_2 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__7; x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__9() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__9() { _start: { lean_object* x_1; @@ -2401,16 +2493,16 @@ x_1 = lean_mk_string_unchecked("unknown '", 9, 9); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__10() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__10() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__9; +x_1 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__9; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__11() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__11() { _start: { lean_object* x_1; @@ -2418,16 +2510,16 @@ x_1 = lean_mk_string_unchecked("' field '", 9, 9); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__12() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__12() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__11; +x_1 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__11; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__13() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__13() { _start: { lean_object* x_1; @@ -2435,16 +2527,16 @@ x_1 = lean_mk_string_unchecked("'", 1, 1); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__14() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__14() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__13; +x_1 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__13; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___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) { _start: { uint8_t x_9; @@ -2471,7 +2563,7 @@ if (x_20 == 0) lean_object* x_21; lean_object* x_22; uint8_t x_23; lean_dec(x_5); lean_dec(x_1); -x_21 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__2; +x_21 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__2; x_22 = l_Lean_throwErrorAt___at_Lake_DSL_elabConfigDecl___spec__1(x_11, x_21, x_6, x_7, x_8); lean_dec(x_11); x_23 = !lean_is_exclusive(x_22); @@ -2501,7 +2593,7 @@ x_28 = l_Lean_Syntax_getArg(x_11, x_27); x_29 = lean_unsigned_to_nat(2u); x_30 = l_Lean_Syntax_getArg(x_11, x_29); x_31 = l_Lean_Syntax_getId(x_28); -x_32 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__8; +x_32 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__8; lean_inc(x_1); lean_inc(x_31); x_33 = lean_alloc_ctor(3, 4, 0); @@ -2538,11 +2630,11 @@ x_44 = lean_box(0); lean_inc(x_1); x_45 = l_Lean_Expr_const___override(x_1, x_44); x_46 = l_Lean_MessageData_ofExpr(x_45); -x_47 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__10; +x_47 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__10; lean_ctor_set_tag(x_38, 7); lean_ctor_set(x_38, 1, x_46); lean_ctor_set(x_38, 0, x_47); -x_48 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__12; +x_48 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__12; lean_ctor_set_tag(x_34, 7); lean_ctor_set(x_34, 1, x_48); lean_ctor_set(x_34, 0, x_38); @@ -2550,7 +2642,7 @@ x_49 = l_Lean_MessageData_ofName(x_31); x_50 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_50, 0, x_34); lean_ctor_set(x_50, 1, x_49); -x_51 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__14; +x_51 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__14; x_52 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_52, 0, x_50); lean_ctor_set(x_52, 1, x_51); @@ -2622,11 +2714,11 @@ x_66 = lean_box(0); lean_inc(x_1); x_67 = l_Lean_Expr_const___override(x_1, x_66); x_68 = l_Lean_MessageData_ofExpr(x_67); -x_69 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__10; +x_69 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__10; x_70 = lean_alloc_ctor(7, 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_Lake_DSL_elabConfigDecl___spec__2___closed__12; +x_71 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__12; lean_ctor_set_tag(x_34, 7); lean_ctor_set(x_34, 1, x_71); lean_ctor_set(x_34, 0, x_70); @@ -2634,7 +2726,7 @@ x_72 = l_Lean_MessageData_ofName(x_31); x_73 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_73, 0, x_34); lean_ctor_set(x_73, 1, x_72); -x_74 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__14; +x_74 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__14; x_75 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_75, 0, x_73); lean_ctor_set(x_75, 1, x_74); @@ -2711,7 +2803,7 @@ x_91 = lean_box(0); lean_inc(x_1); x_92 = l_Lean_Expr_const___override(x_1, x_91); x_93 = l_Lean_MessageData_ofExpr(x_92); -x_94 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__10; +x_94 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__10; if (lean_is_scalar(x_88)) { x_95 = lean_alloc_ctor(7, 2, 0); } else { @@ -2720,7 +2812,7 @@ if (lean_is_scalar(x_88)) { } lean_ctor_set(x_95, 0, x_94); lean_ctor_set(x_95, 1, x_93); -x_96 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__12; +x_96 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__12; x_97 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_97, 0, x_95); lean_ctor_set(x_97, 1, x_96); @@ -2728,7 +2820,7 @@ x_98 = l_Lean_MessageData_ofName(x_31); x_99 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_99, 0, x_97); lean_ctor_set(x_99, 1, x_98); -x_100 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__14; +x_100 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__14; x_101 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_101, 0, x_99); lean_ctor_set(x_101, 1, x_100); @@ -2791,7 +2883,7 @@ goto _start; } } } -static lean_object* _init_l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__1() { +static lean_object* _init_l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__1() { _start: { lean_object* x_1; @@ -2799,19 +2891,19 @@ x_1 = lean_mk_string_unchecked("structInstField", 15, 15); return x_1; } } -static lean_object* _init_l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__2() { +static lean_object* _init_l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lake_DSL_expandAttrs___closed__2; x_2 = l_Lake_DSL_expandAttrs___closed__3; x_3 = l_Lake_DSL_expandAttrs___closed__4; -x_4 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__1; +x_4 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__1; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__3() { +static lean_object* _init_l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__3() { _start: { lean_object* x_1; @@ -2819,19 +2911,19 @@ x_1 = lean_mk_string_unchecked("structInstLVal", 14, 14); return x_1; } } -static lean_object* _init_l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__4() { +static lean_object* _init_l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lake_DSL_expandAttrs___closed__2; x_2 = l_Lake_DSL_expandAttrs___closed__3; x_3 = l_Lake_DSL_expandAttrs___closed__4; -x_4 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__3; +x_4 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__3; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__5() { +static lean_object* _init_l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__5() { _start: { lean_object* x_1; lean_object* x_2; @@ -2840,7 +2932,7 @@ x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -static lean_object* _init_l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6() { +static lean_object* _init_l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6() { _start: { lean_object* x_1; @@ -2848,7 +2940,7 @@ x_1 = lean_mk_string_unchecked(":=", 2, 2); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { if (lean_obj_tag(x_2) == 0) @@ -2871,7 +2963,7 @@ lean_inc(x_9); x_10 = lean_ctor_get(x_2, 3); lean_inc(x_10); lean_dec(x_2); -x_11 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3(x_1, x_7, x_3, x_4, x_5); +x_11 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4(x_1, x_7, x_3, x_4, x_5); x_12 = lean_ctor_get(x_11, 0); lean_inc(x_12); x_13 = lean_ctor_get(x_11, 1); @@ -2952,21 +3044,21 @@ x_44 = lean_ctor_get(x_42, 1); x_45 = lean_ctor_get(x_42, 0); lean_dec(x_45); x_46 = l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__8; -x_47 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__5; +x_47 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__5; lean_inc(x_39); x_48 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_48, 0, x_39); lean_ctor_set(x_48, 1, x_46); lean_ctor_set(x_48, 2, x_47); -x_49 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__4; +x_49 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__4; lean_inc(x_39); x_50 = l_Lean_Syntax_node2(x_39, x_49, x_33, x_48); -x_51 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_51 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_39); lean_ctor_set_tag(x_42, 2); lean_ctor_set(x_42, 1, x_51); lean_ctor_set(x_42, 0, x_39); -x_52 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__2; +x_52 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__2; x_53 = l_Lean_Syntax_node3(x_39, x_52, x_50, x_42, x_15); x_54 = lean_array_push(x_12, x_53); x_1 = x_54; @@ -2981,21 +3073,21 @@ x_56 = lean_ctor_get(x_42, 1); lean_inc(x_56); lean_dec(x_42); x_57 = l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__8; -x_58 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__5; +x_58 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__5; lean_inc(x_39); x_59 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_59, 0, x_39); lean_ctor_set(x_59, 1, x_57); lean_ctor_set(x_59, 2, x_58); -x_60 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__4; +x_60 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__4; lean_inc(x_39); x_61 = l_Lean_Syntax_node2(x_39, x_60, x_33, x_59); -x_62 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_62 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_39); x_63 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_63, 0, x_39); lean_ctor_set(x_63, 1, x_62); -x_64 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__2; +x_64 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__2; x_65 = l_Lean_Syntax_node3(x_39, x_64, x_61, x_63, x_15); x_66 = lean_array_push(x_12, x_65); x_1 = x_66; @@ -3006,7 +3098,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__4(size_t x_1, size_t x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__5(size_t x_1, size_t x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -3030,7 +3122,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__6___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__7___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; uint8_t x_9; @@ -3066,7 +3158,7 @@ return x_15; } } } -static lean_object* _init_l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__6___closed__1() { +static lean_object* _init_l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__7___closed__1() { _start: { lean_object* x_1; @@ -3074,32 +3166,32 @@ x_1 = lean_mk_string_unchecked("x", 1, 1); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__6___closed__2() { +static lean_object* _init_l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__7___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___at_Lake_DSL_elabConfigDecl___spec__6___closed__1; +x_2 = l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__7___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___at_Lake_DSL_elabConfigDecl___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__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; -x_4 = l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__6___closed__2; -x_5 = lean_alloc_closure((void*)(l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__6___lambda__1___boxed), 4, 1); +x_4 = l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__7___closed__2; +x_5 = lean_alloc_closure((void*)(l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__7___lambda__1___boxed), 4, 1); lean_closure_set(x_5, 0, x_4); x_6 = l_Lean_Elab_Command_withFreshMacroScope___rarg(x_5, x_1, x_2, x_3); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshIdent___at_Lake_DSL_elabConfigDecl___spec__5(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_Elab_Term_mkFreshIdent___at_Lake_DSL_elabConfigDecl___spec__6(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; -x_6 = l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__6(x_3, x_4, x_5); +x_6 = l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__7(x_3, x_4, x_5); if (lean_obj_tag(x_6) == 0) { uint8_t x_7; @@ -3151,7 +3243,7 @@ return x_17; } } } -LEAN_EXPORT lean_object* l_Lean_mkIdentFromRef___at_Lake_DSL_elabConfigDecl___spec__7(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_mkIdentFromRef___at_Lake_DSL_elabConfigDecl___spec__8(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; uint8_t x_7; @@ -3183,7 +3275,7 @@ return x_13; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { uint8_t x_11; @@ -3209,7 +3301,7 @@ if (x_21 == 0) lean_object* x_22; lean_object* x_23; uint8_t x_24; lean_dec(x_7); lean_dec(x_1); -x_22 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__2; +x_22 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__2; x_23 = l_Lean_throwErrorAt___at_Lake_DSL_elabConfigDecl___spec__1(x_13, x_22, x_8, x_9, x_10); lean_dec(x_13); x_24 = !lean_is_exclusive(x_23); @@ -3239,7 +3331,7 @@ x_29 = l_Lean_Syntax_getArg(x_13, x_28); x_30 = lean_unsigned_to_nat(2u); x_31 = l_Lean_Syntax_getArg(x_13, x_30); x_32 = l_Lean_Syntax_getId(x_29); -x_33 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__8; +x_33 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__8; lean_inc(x_1); lean_inc(x_32); x_34 = lean_alloc_ctor(3, 4, 0); @@ -3276,11 +3368,11 @@ x_45 = lean_box(0); lean_inc(x_1); x_46 = l_Lean_Expr_const___override(x_1, x_45); x_47 = l_Lean_MessageData_ofExpr(x_46); -x_48 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__10; +x_48 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__10; lean_ctor_set_tag(x_39, 7); lean_ctor_set(x_39, 1, x_47); lean_ctor_set(x_39, 0, x_48); -x_49 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__12; +x_49 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__12; lean_ctor_set_tag(x_35, 7); lean_ctor_set(x_35, 1, x_49); lean_ctor_set(x_35, 0, x_39); @@ -3288,7 +3380,7 @@ x_50 = l_Lean_MessageData_ofName(x_32); x_51 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_51, 0, x_35); lean_ctor_set(x_51, 1, x_50); -x_52 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__14; +x_52 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__14; x_53 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_53, 0, x_51); lean_ctor_set(x_53, 1, x_52); @@ -3360,11 +3452,11 @@ x_67 = lean_box(0); lean_inc(x_1); x_68 = l_Lean_Expr_const___override(x_1, x_67); x_69 = l_Lean_MessageData_ofExpr(x_68); -x_70 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__10; +x_70 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__10; x_71 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_71, 0, x_70); lean_ctor_set(x_71, 1, x_69); -x_72 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__12; +x_72 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__12; lean_ctor_set_tag(x_35, 7); lean_ctor_set(x_35, 1, x_72); lean_ctor_set(x_35, 0, x_71); @@ -3372,7 +3464,7 @@ x_73 = l_Lean_MessageData_ofName(x_32); x_74 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_74, 0, x_35); lean_ctor_set(x_74, 1, x_73); -x_75 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__14; +x_75 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__14; x_76 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_76, 0, x_74); lean_ctor_set(x_76, 1, x_75); @@ -3449,7 +3541,7 @@ x_92 = lean_box(0); lean_inc(x_1); x_93 = l_Lean_Expr_const___override(x_1, x_92); x_94 = l_Lean_MessageData_ofExpr(x_93); -x_95 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__10; +x_95 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__10; if (lean_is_scalar(x_89)) { x_96 = lean_alloc_ctor(7, 2, 0); } else { @@ -3458,7 +3550,7 @@ if (lean_is_scalar(x_89)) { } lean_ctor_set(x_96, 0, x_95); lean_ctor_set(x_96, 1, x_94); -x_97 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__12; +x_97 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__12; x_98 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_98, 0, x_96); lean_ctor_set(x_98, 1, x_97); @@ -3466,7 +3558,7 @@ x_99 = l_Lean_MessageData_ofName(x_32); x_100 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_100, 0, x_98); lean_ctor_set(x_100, 1, x_99); -x_101 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__14; +x_101 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__14; x_102 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_102, 0, x_100); lean_ctor_set(x_102, 1, x_101); @@ -3529,7 +3621,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___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_EXPORT lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { if (lean_obj_tag(x_3) == 0) @@ -3552,7 +3644,7 @@ lean_inc(x_10); x_11 = lean_ctor_get(x_3, 3); lean_inc(x_11); lean_dec(x_3); -x_12 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__9(x_1, x_2, x_8, x_4, x_5, x_6); +x_12 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__10(x_1, x_2, x_8, x_4, x_5, x_6); x_13 = lean_ctor_get(x_12, 0); lean_inc(x_13); x_14 = lean_ctor_get(x_12, 1); @@ -3633,21 +3725,21 @@ x_45 = lean_ctor_get(x_43, 1); x_46 = lean_ctor_get(x_43, 0); lean_dec(x_46); x_47 = l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__8; -x_48 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__5; +x_48 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__5; lean_inc(x_40); x_49 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_49, 0, x_40); lean_ctor_set(x_49, 1, x_47); lean_ctor_set(x_49, 2, x_48); -x_50 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__4; +x_50 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__4; lean_inc(x_40); x_51 = l_Lean_Syntax_node2(x_40, x_50, x_34, x_49); -x_52 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_52 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_40); lean_ctor_set_tag(x_43, 2); lean_ctor_set(x_43, 1, x_52); lean_ctor_set(x_43, 0, x_40); -x_53 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__2; +x_53 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__2; x_54 = l_Lean_Syntax_node3(x_40, x_53, x_51, x_43, x_16); x_55 = lean_array_push(x_13, x_54); x_2 = x_55; @@ -3662,21 +3754,21 @@ x_57 = lean_ctor_get(x_43, 1); lean_inc(x_57); lean_dec(x_43); x_58 = l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__8; -x_59 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__5; +x_59 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__5; lean_inc(x_40); x_60 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_60, 0, x_40); lean_ctor_set(x_60, 1, x_58); lean_ctor_set(x_60, 2, x_59); -x_61 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__4; +x_61 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__4; lean_inc(x_40); x_62 = l_Lean_Syntax_node2(x_40, x_61, x_34, x_60); -x_63 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_63 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_40); x_64 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_64, 0, x_40); lean_ctor_set(x_64, 1, x_63); -x_65 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__2; +x_65 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__2; x_66 = l_Lean_Syntax_node3(x_40, x_65, x_62, x_64, x_16); x_67 = lean_array_push(x_13, x_66); x_2 = x_67; @@ -3687,7 +3779,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_sequenceMap_loop___at_Lake_DSL_elabConfigDecl___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_Array_sequenceMap_loop___at_Lake_DSL_elabConfigDecl___spec__12(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; @@ -3756,18 +3848,18 @@ return x_20; } } } -LEAN_EXPORT lean_object* l_Array_sequenceMap___at_Lake_DSL_elabConfigDecl___spec__10(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_sequenceMap___at_Lake_DSL_elabConfigDecl___spec__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; x_3 = lean_array_get_size(x_1); x_4 = lean_mk_empty_array_with_capacity(x_3); x_5 = lean_unsigned_to_nat(0u); -x_6 = l_Array_sequenceMap_loop___at_Lake_DSL_elabConfigDecl___spec__11(x_1, x_2, x_3, x_5, x_4); +x_6 = l_Array_sequenceMap_loop___at_Lake_DSL_elabConfigDecl___spec__12(x_1, x_2, x_3, x_5, x_4); return x_6; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__12(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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__13(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) { _start: { uint8_t x_10; @@ -3794,7 +3886,7 @@ if (x_21 == 0) lean_object* x_22; lean_object* x_23; uint8_t x_24; lean_dec(x_6); lean_dec(x_1); -x_22 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__2; +x_22 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__2; x_23 = l_Lean_throwErrorAt___at_Lake_DSL_elabConfigDecl___spec__1(x_12, x_22, x_7, x_8, x_9); lean_dec(x_12); x_24 = !lean_is_exclusive(x_23); @@ -3824,7 +3916,7 @@ x_29 = l_Lean_Syntax_getArg(x_12, x_28); x_30 = lean_unsigned_to_nat(2u); x_31 = l_Lean_Syntax_getArg(x_12, x_30); x_32 = l_Lean_Syntax_getId(x_29); -x_33 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__8; +x_33 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__8; lean_inc(x_1); lean_inc(x_32); x_34 = lean_alloc_ctor(3, 4, 0); @@ -3861,11 +3953,11 @@ x_45 = lean_box(0); lean_inc(x_1); x_46 = l_Lean_Expr_const___override(x_1, x_45); x_47 = l_Lean_MessageData_ofExpr(x_46); -x_48 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__10; +x_48 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__10; lean_ctor_set_tag(x_39, 7); lean_ctor_set(x_39, 1, x_47); lean_ctor_set(x_39, 0, x_48); -x_49 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__12; +x_49 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__12; lean_ctor_set_tag(x_35, 7); lean_ctor_set(x_35, 1, x_49); lean_ctor_set(x_35, 0, x_39); @@ -3873,7 +3965,7 @@ x_50 = l_Lean_MessageData_ofName(x_32); x_51 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_51, 0, x_35); lean_ctor_set(x_51, 1, x_50); -x_52 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__14; +x_52 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__14; x_53 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_53, 0, x_51); lean_ctor_set(x_53, 1, x_52); @@ -3945,11 +4037,11 @@ x_67 = lean_box(0); lean_inc(x_1); x_68 = l_Lean_Expr_const___override(x_1, x_67); x_69 = l_Lean_MessageData_ofExpr(x_68); -x_70 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__10; +x_70 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__10; x_71 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_71, 0, x_70); lean_ctor_set(x_71, 1, x_69); -x_72 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__12; +x_72 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__12; lean_ctor_set_tag(x_35, 7); lean_ctor_set(x_35, 1, x_72); lean_ctor_set(x_35, 0, x_71); @@ -3957,7 +4049,7 @@ x_73 = l_Lean_MessageData_ofName(x_32); x_74 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_74, 0, x_35); lean_ctor_set(x_74, 1, x_73); -x_75 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__14; +x_75 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__14; x_76 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_76, 0, x_74); lean_ctor_set(x_76, 1, x_75); @@ -4034,7 +4126,7 @@ x_92 = lean_box(0); lean_inc(x_1); x_93 = l_Lean_Expr_const___override(x_1, x_92); x_94 = l_Lean_MessageData_ofExpr(x_93); -x_95 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__10; +x_95 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__10; if (lean_is_scalar(x_89)) { x_96 = lean_alloc_ctor(7, 2, 0); } else { @@ -4043,7 +4135,7 @@ if (lean_is_scalar(x_89)) { } lean_ctor_set(x_96, 0, x_95); lean_ctor_set(x_96, 1, x_94); -x_97 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__12; +x_97 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__12; x_98 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_98, 0, x_96); lean_ctor_set(x_98, 1, x_97); @@ -4051,7 +4143,7 @@ x_99 = l_Lean_MessageData_ofName(x_32); x_100 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_100, 0, x_98); lean_ctor_set(x_100, 1, x_99); -x_101 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__14; +x_101 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__14; x_102 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_102, 0, x_100); lean_ctor_set(x_102, 1, x_101); @@ -4114,7 +4206,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___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_EXPORT lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___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) { _start: { if (lean_obj_tag(x_3) == 0) @@ -4137,7 +4229,7 @@ lean_inc(x_10); x_11 = lean_ctor_get(x_3, 3); lean_inc(x_11); lean_dec(x_3); -x_12 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__13(x_1, x_2, x_8, x_4, x_5, x_6); +x_12 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__14(x_1, x_2, x_8, x_4, x_5, x_6); x_13 = lean_ctor_get(x_12, 0); lean_inc(x_13); x_14 = lean_ctor_get(x_12, 1); @@ -4218,21 +4310,21 @@ x_45 = lean_ctor_get(x_43, 1); x_46 = lean_ctor_get(x_43, 0); lean_dec(x_46); x_47 = l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__8; -x_48 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__5; +x_48 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__5; lean_inc(x_40); x_49 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_49, 0, x_40); lean_ctor_set(x_49, 1, x_47); lean_ctor_set(x_49, 2, x_48); -x_50 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__4; +x_50 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__4; lean_inc(x_40); x_51 = l_Lean_Syntax_node2(x_40, x_50, x_34, x_49); -x_52 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_52 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_40); lean_ctor_set_tag(x_43, 2); lean_ctor_set(x_43, 1, x_52); lean_ctor_set(x_43, 0, x_40); -x_53 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__2; +x_53 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__2; x_54 = l_Lean_Syntax_node3(x_40, x_53, x_51, x_43, x_16); x_55 = lean_array_push(x_13, x_54); x_2 = x_55; @@ -4247,21 +4339,21 @@ x_57 = lean_ctor_get(x_43, 1); lean_inc(x_57); lean_dec(x_43); x_58 = l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__8; -x_59 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__5; +x_59 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__5; lean_inc(x_40); x_60 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_60, 0, x_40); lean_ctor_set(x_60, 1, x_58); lean_ctor_set(x_60, 2, x_59); -x_61 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__4; +x_61 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__4; lean_inc(x_40); x_62 = l_Lean_Syntax_node2(x_40, x_61, x_34, x_60); -x_63 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_63 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_40); x_64 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_64, 0, x_40); lean_ctor_set(x_64, 1, x_63); -x_65 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__2; +x_65 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__2; x_66 = l_Lean_Syntax_node3(x_40, x_65, x_62, x_64, x_16); x_67 = lean_array_push(x_13, x_66); x_2 = x_67; @@ -4486,7 +4578,7 @@ static lean_object* _init_l_Lake_DSL_elabConfigDecl___lambda__2___closed__20() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__5; +x_1 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__5; x_2 = l_Array_append___rarg(x_1, x_1); return x_2; } @@ -4545,7 +4637,7 @@ x_15 = lean_array_size(x_1); x_16 = 0; lean_inc(x_12); lean_inc(x_2); -x_17 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2(x_2, x_1, x_15, x_16, x_10, x_12, x_13, x_14); +x_17 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3(x_2, x_1, x_15, x_16, x_10, x_12, x_13, x_14); if (lean_obj_tag(x_17) == 0) { lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; @@ -4555,7 +4647,7 @@ x_19 = lean_ctor_get(x_17, 1); lean_inc(x_19); lean_dec(x_17); x_20 = l_Lake_DSL_expandAttrs___closed__1; -x_21 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3(x_20, x_18, x_12, x_13, x_19); +x_21 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4(x_20, x_18, x_12, x_13, x_19); x_22 = lean_ctor_get(x_21, 0); lean_inc(x_22); x_23 = lean_ctor_get(x_21, 1); @@ -4586,7 +4678,7 @@ x_677 = lean_ctor_get(x_675, 0); x_678 = lean_ctor_get(x_675, 1); lean_inc(x_13); lean_inc(x_12); -x_679 = l_Lean_Elab_Term_mkFreshIdent___at_Lake_DSL_elabConfigDecl___spec__5(x_677, x_28, x_12, x_13, x_678); +x_679 = l_Lean_Elab_Term_mkFreshIdent___at_Lake_DSL_elabConfigDecl___spec__6(x_677, x_28, x_12, x_13, x_678); lean_dec(x_677); if (lean_obj_tag(x_679) == 0) { @@ -4652,7 +4744,7 @@ lean_inc(x_691); lean_dec(x_675); lean_inc(x_13); lean_inc(x_12); -x_693 = l_Lean_Elab_Term_mkFreshIdent___at_Lake_DSL_elabConfigDecl___spec__5(x_691, x_28, x_12, x_13, x_692); +x_693 = l_Lean_Elab_Term_mkFreshIdent___at_Lake_DSL_elabConfigDecl___spec__6(x_691, x_28, x_12, x_13, x_692); lean_dec(x_691); if (lean_obj_tag(x_693) == 0) { @@ -4716,7 +4808,7 @@ lean_object* x_706; lean_object* x_707; uint8_t x_708; x_706 = lean_ctor_get(x_9, 0); lean_inc(x_706); lean_dec(x_9); -x_707 = l_Lean_mkIdentFromRef___at_Lake_DSL_elabConfigDecl___spec__7(x_706, x_28, x_12, x_13, x_27); +x_707 = l_Lean_mkIdentFromRef___at_Lake_DSL_elabConfigDecl___spec__8(x_706, x_28, x_12, x_13, x_27); x_708 = !lean_is_exclusive(x_707); if (x_708 == 0) { @@ -4882,14 +4974,14 @@ lean_ctor_set_tag(x_57, 2); lean_ctor_set(x_57, 1, x_61); lean_ctor_set(x_57, 0, x_52); x_62 = l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__8; -x_63 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__5; +x_63 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__5; lean_inc(x_52); x_64 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_64, 0, x_52); lean_ctor_set(x_64, 1, x_62); lean_ctor_set(x_64, 2, x_63); x_65 = lean_array_size(x_22); -x_66 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__4(x_65, x_16, x_22); +x_66 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__5(x_65, x_16, x_22); x_67 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__4; x_68 = l_Lean_mkSepArray(x_66, x_67); lean_dec(x_66); @@ -4985,7 +5077,7 @@ x_104 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__16; lean_inc(x_98); lean_inc(x_80); x_105 = l_Lean_Syntax_node2(x_80, x_104, x_98, x_103); -x_106 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_106 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_80); lean_ctor_set_tag(x_32, 2); lean_ctor_set(x_32, 1, x_106); @@ -5130,7 +5222,7 @@ x_156 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__16; lean_inc(x_150); lean_inc(x_80); x_157 = l_Lean_Syntax_node2(x_80, x_156, x_150, x_155); -x_158 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_158 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_80); lean_ctor_set_tag(x_32, 2); lean_ctor_set(x_32, 1, x_158); @@ -5292,7 +5384,7 @@ x_212 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__16; lean_inc(x_206); lean_inc(x_80); x_213 = l_Lean_Syntax_node2(x_80, x_212, x_206, x_211); -x_214 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_214 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_80); lean_ctor_set_tag(x_32, 2); lean_ctor_set(x_32, 1, x_214); @@ -5474,7 +5566,7 @@ x_274 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__16; lean_inc(x_267); lean_inc(x_249); x_275 = l_Lean_Syntax_node2(x_249, x_274, x_267, x_273); -x_276 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_276 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_249); lean_ctor_set_tag(x_32, 2); lean_ctor_set(x_32, 1, x_276); @@ -5578,14 +5670,14 @@ x_311 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_311, 0, x_52); lean_ctor_set(x_311, 1, x_310); x_312 = l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__8; -x_313 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__5; +x_313 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__5; lean_inc(x_52); x_314 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_314, 0, x_52); lean_ctor_set(x_314, 1, x_312); lean_ctor_set(x_314, 2, x_313); x_315 = lean_array_size(x_22); -x_316 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__4(x_315, x_16, x_22); +x_316 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__5(x_315, x_16, x_22); x_317 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__4; x_318 = l_Lean_mkSepArray(x_316, x_317); lean_dec(x_316); @@ -5708,7 +5800,7 @@ x_355 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__16; lean_inc(x_348); lean_inc(x_330); x_356 = l_Lean_Syntax_node2(x_330, x_355, x_348, x_354); -x_357 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_357 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_330); lean_ctor_set_tag(x_32, 2); lean_ctor_set(x_32, 1, x_357); @@ -5828,14 +5920,14 @@ if (lean_is_scalar(x_393)) { lean_ctor_set(x_395, 0, x_52); lean_ctor_set(x_395, 1, x_394); x_396 = l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__8; -x_397 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__5; +x_397 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__5; lean_inc(x_52); x_398 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_398, 0, x_52); lean_ctor_set(x_398, 1, x_396); lean_ctor_set(x_398, 2, x_397); x_399 = lean_array_size(x_22); -x_400 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__4(x_399, x_16, x_22); +x_400 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__5(x_399, x_16, x_22); x_401 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__4; x_402 = l_Lean_mkSepArray(x_400, x_401); lean_dec(x_400); @@ -5958,7 +6050,7 @@ x_440 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__16; lean_inc(x_433); lean_inc(x_415); x_441 = l_Lean_Syntax_node2(x_415, x_440, x_433, x_439); -x_442 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_442 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_415); lean_ctor_set_tag(x_32, 2); lean_ctor_set(x_32, 1, x_442); @@ -6094,14 +6186,14 @@ if (lean_is_scalar(x_483)) { lean_ctor_set(x_485, 0, x_477); lean_ctor_set(x_485, 1, x_484); x_486 = l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__8; -x_487 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__5; +x_487 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__5; lean_inc(x_477); x_488 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_488, 0, x_477); lean_ctor_set(x_488, 1, x_486); lean_ctor_set(x_488, 2, x_487); x_489 = lean_array_size(x_22); -x_490 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__4(x_489, x_16, x_22); +x_490 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__5(x_489, x_16, x_22); x_491 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__4; x_492 = l_Lean_mkSepArray(x_490, x_491); lean_dec(x_490); @@ -6229,7 +6321,7 @@ x_531 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__16; lean_inc(x_523); lean_inc(x_505); x_532 = l_Lean_Syntax_node2(x_505, x_531, x_523, x_530); -x_533 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_533 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_505); lean_ctor_set_tag(x_32, 2); lean_ctor_set(x_32, 1, x_533); @@ -6411,14 +6503,14 @@ if (lean_is_scalar(x_590)) { lean_ctor_set(x_592, 0, x_584); lean_ctor_set(x_592, 1, x_591); x_593 = l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__8; -x_594 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__5; +x_594 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__5; lean_inc(x_584); x_595 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_595, 0, x_584); lean_ctor_set(x_595, 1, x_593); lean_ctor_set(x_595, 2, x_594); x_596 = lean_array_size(x_22); -x_597 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__4(x_596, x_16, x_22); +x_597 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__5(x_596, x_16, x_22); x_598 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__4; x_599 = l_Lean_mkSepArray(x_597, x_598); lean_dec(x_597); @@ -6551,7 +6643,7 @@ x_638 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__16; lean_inc(x_630); lean_inc(x_612); x_639 = l_Lean_Syntax_node2(x_612, x_638, x_630, x_637); -x_640 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_640 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_612); x_641 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_641, 0, x_612); @@ -6675,7 +6767,7 @@ if (lean_is_exclusive(x_854)) { } lean_inc(x_13); lean_inc(x_12); -x_858 = l_Lean_Elab_Term_mkFreshIdent___at_Lake_DSL_elabConfigDecl___spec__5(x_855, x_739, x_12, x_13, x_856); +x_858 = l_Lean_Elab_Term_mkFreshIdent___at_Lake_DSL_elabConfigDecl___spec__6(x_855, x_739, x_12, x_13, x_856); lean_dec(x_855); if (lean_obj_tag(x_858) == 0) { @@ -6744,7 +6836,7 @@ lean_object* x_871; lean_object* x_872; lean_object* x_873; lean_object* x_874; x_871 = lean_ctor_get(x_9, 0); lean_inc(x_871); lean_dec(x_9); -x_872 = l_Lean_mkIdentFromRef___at_Lake_DSL_elabConfigDecl___spec__7(x_871, x_739, x_12, x_13, x_738); +x_872 = l_Lean_mkIdentFromRef___at_Lake_DSL_elabConfigDecl___spec__8(x_871, x_739, x_12, x_13, x_738); x_873 = lean_ctor_get(x_872, 0); lean_inc(x_873); x_874 = lean_ctor_get(x_872, 1); @@ -6922,14 +7014,14 @@ if (lean_is_scalar(x_769)) { lean_ctor_set(x_771, 0, x_763); lean_ctor_set(x_771, 1, x_770); x_772 = l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__8; -x_773 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__5; +x_773 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__5; lean_inc(x_763); x_774 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_774, 0, x_763); lean_ctor_set(x_774, 1, x_772); lean_ctor_set(x_774, 2, x_773); x_775 = lean_array_size(x_22); -x_776 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__4(x_775, x_16, x_22); +x_776 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__5(x_775, x_16, x_22); x_777 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__4; x_778 = l_Lean_mkSepArray(x_776, x_777); lean_dec(x_776); @@ -7062,7 +7154,7 @@ x_817 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__16; lean_inc(x_809); lean_inc(x_791); x_818 = l_Lean_Syntax_node2(x_791, x_817, x_809, x_816); -x_819 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_819 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_791); if (lean_is_scalar(x_746)) { x_820 = lean_alloc_ctor(2, 2, 0); @@ -7284,7 +7376,7 @@ x_17 = lean_array_size(x_1); x_18 = 0; lean_inc(x_14); lean_inc(x_2); -x_19 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__8(x_2, x_3, x_4, x_1, x_17, x_18, x_12, x_14, x_15, x_16); +x_19 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__9(x_2, x_3, x_4, x_1, x_17, x_18, x_12, x_14, x_15, x_16); if (lean_obj_tag(x_19) == 0) { lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; @@ -7296,7 +7388,7 @@ lean_dec(x_19); lean_inc(x_4); x_22 = lean_array_mk(x_4); lean_inc(x_22); -x_23 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__9(x_4, x_22, x_20, x_14, x_15, x_21); +x_23 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__10(x_4, x_22, x_20, x_14, x_15, x_21); x_24 = !lean_is_exclusive(x_23); if (x_24 == 0) { @@ -7328,7 +7420,7 @@ x_680 = lean_ctor_get(x_678, 0); x_681 = lean_ctor_get(x_678, 1); lean_inc(x_15); lean_inc(x_14); -x_682 = l_Lean_Elab_Term_mkFreshIdent___at_Lake_DSL_elabConfigDecl___spec__5(x_680, x_31, x_14, x_15, x_681); +x_682 = l_Lean_Elab_Term_mkFreshIdent___at_Lake_DSL_elabConfigDecl___spec__6(x_680, x_31, x_14, x_15, x_681); lean_dec(x_680); if (lean_obj_tag(x_682) == 0) { @@ -7404,7 +7496,7 @@ lean_inc(x_695); lean_dec(x_678); lean_inc(x_15); lean_inc(x_14); -x_697 = l_Lean_Elab_Term_mkFreshIdent___at_Lake_DSL_elabConfigDecl___spec__5(x_695, x_31, x_14, x_15, x_696); +x_697 = l_Lean_Elab_Term_mkFreshIdent___at_Lake_DSL_elabConfigDecl___spec__6(x_695, x_31, x_14, x_15, x_696); lean_dec(x_695); if (lean_obj_tag(x_697) == 0) { @@ -7478,7 +7570,7 @@ lean_object* x_711; lean_object* x_712; uint8_t x_713; x_711 = lean_ctor_get(x_11, 0); lean_inc(x_711); lean_dec(x_11); -x_712 = l_Lean_mkIdentFromRef___at_Lake_DSL_elabConfigDecl___spec__7(x_711, x_31, x_14, x_15, x_30); +x_712 = l_Lean_mkIdentFromRef___at_Lake_DSL_elabConfigDecl___spec__8(x_711, x_31, x_14, x_15, x_30); x_713 = !lean_is_exclusive(x_712); if (x_713 == 0) { @@ -7674,14 +7766,14 @@ lean_ctor_set_tag(x_60, 2); lean_ctor_set(x_60, 1, x_64); lean_ctor_set(x_60, 0, x_55); x_65 = l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__8; -x_66 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__5; +x_66 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__5; lean_inc(x_55); x_67 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_67, 0, x_55); lean_ctor_set(x_67, 1, x_65); lean_ctor_set(x_67, 2, x_66); x_68 = lean_array_size(x_25); -x_69 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__4(x_68, x_18, x_25); +x_69 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__5(x_68, x_18, x_25); x_70 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__4; x_71 = l_Lean_mkSepArray(x_69, x_70); lean_dec(x_69); @@ -7777,7 +7869,7 @@ x_107 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__16; lean_inc(x_101); lean_inc(x_83); x_108 = l_Lean_Syntax_node2(x_83, x_107, x_101, x_106); -x_109 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_109 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_83); lean_ctor_set_tag(x_35, 2); lean_ctor_set(x_35, 1, x_109); @@ -7922,7 +8014,7 @@ x_159 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__16; lean_inc(x_153); lean_inc(x_83); x_160 = l_Lean_Syntax_node2(x_83, x_159, x_153, x_158); -x_161 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_161 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_83); lean_ctor_set_tag(x_35, 2); lean_ctor_set(x_35, 1, x_161); @@ -8084,7 +8176,7 @@ x_215 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__16; lean_inc(x_209); lean_inc(x_83); x_216 = l_Lean_Syntax_node2(x_83, x_215, x_209, x_214); -x_217 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_217 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_83); lean_ctor_set_tag(x_35, 2); lean_ctor_set(x_35, 1, x_217); @@ -8266,7 +8358,7 @@ x_277 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__16; lean_inc(x_270); lean_inc(x_252); x_278 = l_Lean_Syntax_node2(x_252, x_277, x_270, x_276); -x_279 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_279 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_252); lean_ctor_set_tag(x_35, 2); lean_ctor_set(x_35, 1, x_279); @@ -8370,14 +8462,14 @@ x_314 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_314, 0, x_55); lean_ctor_set(x_314, 1, x_313); x_315 = l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__8; -x_316 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__5; +x_316 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__5; lean_inc(x_55); x_317 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_317, 0, x_55); lean_ctor_set(x_317, 1, x_315); lean_ctor_set(x_317, 2, x_316); x_318 = lean_array_size(x_25); -x_319 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__4(x_318, x_18, x_25); +x_319 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__5(x_318, x_18, x_25); x_320 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__4; x_321 = l_Lean_mkSepArray(x_319, x_320); lean_dec(x_319); @@ -8500,7 +8592,7 @@ x_358 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__16; lean_inc(x_351); lean_inc(x_333); x_359 = l_Lean_Syntax_node2(x_333, x_358, x_351, x_357); -x_360 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_360 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_333); lean_ctor_set_tag(x_35, 2); lean_ctor_set(x_35, 1, x_360); @@ -8620,14 +8712,14 @@ if (lean_is_scalar(x_396)) { lean_ctor_set(x_398, 0, x_55); lean_ctor_set(x_398, 1, x_397); x_399 = l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__8; -x_400 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__5; +x_400 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__5; lean_inc(x_55); x_401 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_401, 0, x_55); lean_ctor_set(x_401, 1, x_399); lean_ctor_set(x_401, 2, x_400); x_402 = lean_array_size(x_25); -x_403 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__4(x_402, x_18, x_25); +x_403 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__5(x_402, x_18, x_25); x_404 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__4; x_405 = l_Lean_mkSepArray(x_403, x_404); lean_dec(x_403); @@ -8750,7 +8842,7 @@ x_443 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__16; lean_inc(x_436); lean_inc(x_418); x_444 = l_Lean_Syntax_node2(x_418, x_443, x_436, x_442); -x_445 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_445 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_418); lean_ctor_set_tag(x_35, 2); lean_ctor_set(x_35, 1, x_445); @@ -8886,14 +8978,14 @@ if (lean_is_scalar(x_486)) { lean_ctor_set(x_488, 0, x_480); lean_ctor_set(x_488, 1, x_487); x_489 = l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__8; -x_490 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__5; +x_490 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__5; lean_inc(x_480); x_491 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_491, 0, x_480); lean_ctor_set(x_491, 1, x_489); lean_ctor_set(x_491, 2, x_490); x_492 = lean_array_size(x_25); -x_493 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__4(x_492, x_18, x_25); +x_493 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__5(x_492, x_18, x_25); x_494 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__4; x_495 = l_Lean_mkSepArray(x_493, x_494); lean_dec(x_493); @@ -9021,7 +9113,7 @@ x_534 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__16; lean_inc(x_526); lean_inc(x_508); x_535 = l_Lean_Syntax_node2(x_508, x_534, x_526, x_533); -x_536 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_536 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_508); lean_ctor_set_tag(x_35, 2); lean_ctor_set(x_35, 1, x_536); @@ -9203,14 +9295,14 @@ if (lean_is_scalar(x_593)) { lean_ctor_set(x_595, 0, x_587); lean_ctor_set(x_595, 1, x_594); x_596 = l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__8; -x_597 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__5; +x_597 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__5; lean_inc(x_587); x_598 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_598, 0, x_587); lean_ctor_set(x_598, 1, x_596); lean_ctor_set(x_598, 2, x_597); x_599 = lean_array_size(x_25); -x_600 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__4(x_599, x_18, x_25); +x_600 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__5(x_599, x_18, x_25); x_601 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__4; x_602 = l_Lean_mkSepArray(x_600, x_601); lean_dec(x_600); @@ -9343,7 +9435,7 @@ x_641 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__16; lean_inc(x_633); lean_inc(x_615); x_642 = l_Lean_Syntax_node2(x_615, x_641, x_633, x_640); -x_643 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_643 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_615); x_644 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_644, 0, x_615); @@ -9468,7 +9560,7 @@ if (lean_is_exclusive(x_864)) { } lean_inc(x_15); lean_inc(x_14); -x_868 = l_Lean_Elab_Term_mkFreshIdent___at_Lake_DSL_elabConfigDecl___spec__5(x_865, x_749, x_14, x_15, x_866); +x_868 = l_Lean_Elab_Term_mkFreshIdent___at_Lake_DSL_elabConfigDecl___spec__6(x_865, x_749, x_14, x_15, x_866); lean_dec(x_865); if (lean_obj_tag(x_868) == 0) { @@ -9546,7 +9638,7 @@ lean_object* x_883; lean_object* x_884; lean_object* x_885; lean_object* x_886; x_883 = lean_ctor_get(x_11, 0); lean_inc(x_883); lean_dec(x_11); -x_884 = l_Lean_mkIdentFromRef___at_Lake_DSL_elabConfigDecl___spec__7(x_883, x_749, x_14, x_15, x_748); +x_884 = l_Lean_mkIdentFromRef___at_Lake_DSL_elabConfigDecl___spec__8(x_883, x_749, x_14, x_15, x_748); x_885 = lean_ctor_get(x_884, 0); lean_inc(x_885); x_886 = lean_ctor_get(x_884, 1); @@ -9745,14 +9837,14 @@ if (lean_is_scalar(x_779)) { lean_ctor_set(x_781, 0, x_773); lean_ctor_set(x_781, 1, x_780); x_782 = l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__8; -x_783 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__5; +x_783 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__5; lean_inc(x_773); x_784 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_784, 0, x_773); lean_ctor_set(x_784, 1, x_782); lean_ctor_set(x_784, 2, x_783); x_785 = lean_array_size(x_25); -x_786 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__4(x_785, x_18, x_25); +x_786 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__5(x_785, x_18, x_25); x_787 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__4; x_788 = l_Lean_mkSepArray(x_786, x_787); lean_dec(x_786); @@ -9885,7 +9977,7 @@ x_827 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__16; lean_inc(x_819); lean_inc(x_801); x_828 = l_Lean_Syntax_node2(x_801, x_827, x_819, x_826); -x_829 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_829 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_801); if (lean_is_scalar(x_756)) { x_830 = lean_alloc_ctor(2, 2, 0); @@ -10027,7 +10119,7 @@ if (lean_is_exclusive(x_1035)) { } lean_inc(x_15); lean_inc(x_14); -x_1039 = l_Lean_Elab_Term_mkFreshIdent___at_Lake_DSL_elabConfigDecl___spec__5(x_1036, x_920, x_14, x_15, x_1037); +x_1039 = l_Lean_Elab_Term_mkFreshIdent___at_Lake_DSL_elabConfigDecl___spec__6(x_1036, x_920, x_14, x_15, x_1037); lean_dec(x_1036); if (lean_obj_tag(x_1039) == 0) { @@ -10111,7 +10203,7 @@ lean_object* x_1054; lean_object* x_1055; lean_object* x_1056; lean_object* x_10 x_1054 = lean_ctor_get(x_11, 0); lean_inc(x_1054); lean_dec(x_11); -x_1055 = l_Lean_mkIdentFromRef___at_Lake_DSL_elabConfigDecl___spec__7(x_1054, x_920, x_14, x_15, x_918); +x_1055 = l_Lean_mkIdentFromRef___at_Lake_DSL_elabConfigDecl___spec__8(x_1054, x_920, x_14, x_15, x_918); x_1056 = lean_ctor_get(x_1055, 0); lean_inc(x_1056); x_1057 = lean_ctor_get(x_1055, 1); @@ -10325,14 +10417,14 @@ if (lean_is_scalar(x_950)) { lean_ctor_set(x_952, 0, x_944); lean_ctor_set(x_952, 1, x_951); x_953 = l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__8; -x_954 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__5; +x_954 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__5; lean_inc(x_944); x_955 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_955, 0, x_944); lean_ctor_set(x_955, 1, x_953); lean_ctor_set(x_955, 2, x_954); x_956 = lean_array_size(x_914); -x_957 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__4(x_956, x_18, x_914); +x_957 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__5(x_956, x_18, x_914); x_958 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__4; x_959 = l_Lean_mkSepArray(x_957, x_958); lean_dec(x_957); @@ -10465,7 +10557,7 @@ x_998 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__16; lean_inc(x_990); lean_inc(x_972); x_999 = l_Lean_Syntax_node2(x_972, x_998, x_990, x_997); -x_1000 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_1000 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_972); if (lean_is_scalar(x_927)) { x_1001 = lean_alloc_ctor(2, 2, 0); @@ -10820,7 +10912,7 @@ x_30 = l_Lean_Syntax_getArgs(x_29); lean_dec(x_29); x_31 = lean_alloc_closure((void*)(l_Lake_DSL_elabConfigDecl___lambda__7___boxed), 2, 1); lean_closure_set(x_31, 0, x_3); -x_32 = l_Array_sequenceMap___at_Lake_DSL_elabConfigDecl___spec__10(x_30, x_31); +x_32 = l_Array_sequenceMap___at_Lake_DSL_elabConfigDecl___spec__11(x_30, x_31); lean_dec(x_30); if (lean_obj_tag(x_32) == 0) { @@ -11130,7 +11222,7 @@ x_29 = l_Lean_Syntax_getArgs(x_28); lean_dec(x_28); x_30 = lean_alloc_closure((void*)(l_Lake_DSL_elabConfigDecl___lambda__7___boxed), 2, 1); lean_closure_set(x_30, 0, x_3); -x_31 = l_Array_sequenceMap___at_Lake_DSL_elabConfigDecl___spec__10(x_29, x_30); +x_31 = l_Array_sequenceMap___at_Lake_DSL_elabConfigDecl___spec__11(x_29, x_30); lean_dec(x_29); if (lean_obj_tag(x_31) == 0) { @@ -11375,7 +11467,7 @@ x_15 = lean_array_size(x_1); x_16 = 0; lean_inc(x_12); lean_inc(x_2); -x_17 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__12(x_2, x_3, x_1, x_15, x_16, x_10, x_12, x_13, x_14); +x_17 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__13(x_2, x_3, x_1, x_15, x_16, x_10, x_12, x_13, x_14); if (lean_obj_tag(x_17) == 0) { lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; @@ -11385,7 +11477,7 @@ x_19 = lean_ctor_get(x_17, 1); lean_inc(x_19); lean_dec(x_17); lean_inc(x_1); -x_20 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__13(x_3, x_1, x_18, x_12, x_13, x_19); +x_20 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__14(x_3, x_1, x_18, x_12, x_13, x_19); x_21 = !lean_is_exclusive(x_20); if (x_21 == 0) { @@ -11532,14 +11624,14 @@ lean_ctor_set_tag(x_57, 2); lean_ctor_set(x_57, 1, x_61); lean_ctor_set(x_57, 0, x_52); x_62 = l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__8; -x_63 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__5; +x_63 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__5; lean_inc(x_52); x_64 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_64, 0, x_52); lean_ctor_set(x_64, 1, x_62); lean_ctor_set(x_64, 2, x_63); x_65 = lean_array_size(x_22); -x_66 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__4(x_65, x_16, x_22); +x_66 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__5(x_65, x_16, x_22); x_67 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__4; x_68 = l_Lean_mkSepArray(x_66, x_67); lean_dec(x_66); @@ -11635,7 +11727,7 @@ x_104 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__16; lean_inc(x_98); lean_inc(x_80); x_105 = l_Lean_Syntax_node2(x_80, x_104, x_98, x_103); -x_106 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_106 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_80); lean_ctor_set_tag(x_32, 2); lean_ctor_set(x_32, 1, x_106); @@ -11754,7 +11846,7 @@ x_148 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__16; lean_inc(x_142); lean_inc(x_80); x_149 = l_Lean_Syntax_node2(x_80, x_148, x_142, x_147); -x_150 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_150 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_80); lean_ctor_set_tag(x_32, 2); lean_ctor_set(x_32, 1, x_150); @@ -11890,7 +11982,7 @@ x_196 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__16; lean_inc(x_190); lean_inc(x_80); x_197 = l_Lean_Syntax_node2(x_80, x_196, x_190, x_195); -x_198 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_198 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_80); lean_ctor_set_tag(x_32, 2); lean_ctor_set(x_32, 1, x_198); @@ -12046,7 +12138,7 @@ x_250 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__16; lean_inc(x_243); lean_inc(x_225); x_251 = l_Lean_Syntax_node2(x_225, x_250, x_243, x_249); -x_252 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_252 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_225); lean_ctor_set_tag(x_32, 2); lean_ctor_set(x_32, 1, x_252); @@ -12124,14 +12216,14 @@ x_279 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_279, 0, x_52); lean_ctor_set(x_279, 1, x_278); x_280 = l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__8; -x_281 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__5; +x_281 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__5; lean_inc(x_52); x_282 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_282, 0, x_52); lean_ctor_set(x_282, 1, x_280); lean_ctor_set(x_282, 2, x_281); x_283 = lean_array_size(x_22); -x_284 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__4(x_283, x_16, x_22); +x_284 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__5(x_283, x_16, x_22); x_285 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__4; x_286 = l_Lean_mkSepArray(x_284, x_285); lean_dec(x_284); @@ -12254,7 +12346,7 @@ x_323 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__16; lean_inc(x_316); lean_inc(x_298); x_324 = l_Lean_Syntax_node2(x_298, x_323, x_316, x_322); -x_325 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_325 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_298); lean_ctor_set_tag(x_32, 2); lean_ctor_set(x_32, 1, x_325); @@ -12348,14 +12440,14 @@ if (lean_is_scalar(x_353)) { lean_ctor_set(x_355, 0, x_52); lean_ctor_set(x_355, 1, x_354); x_356 = l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__8; -x_357 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__5; +x_357 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__5; lean_inc(x_52); x_358 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_358, 0, x_52); lean_ctor_set(x_358, 1, x_356); lean_ctor_set(x_358, 2, x_357); x_359 = lean_array_size(x_22); -x_360 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__4(x_359, x_16, x_22); +x_360 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__5(x_359, x_16, x_22); x_361 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__4; x_362 = l_Lean_mkSepArray(x_360, x_361); lean_dec(x_360); @@ -12478,7 +12570,7 @@ x_400 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__16; lean_inc(x_393); lean_inc(x_375); x_401 = l_Lean_Syntax_node2(x_375, x_400, x_393, x_399); -x_402 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_402 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_375); lean_ctor_set_tag(x_32, 2); lean_ctor_set(x_32, 1, x_402); @@ -12588,14 +12680,14 @@ if (lean_is_scalar(x_435)) { lean_ctor_set(x_437, 0, x_429); lean_ctor_set(x_437, 1, x_436); x_438 = l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__8; -x_439 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__5; +x_439 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__5; lean_inc(x_429); x_440 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_440, 0, x_429); lean_ctor_set(x_440, 1, x_438); lean_ctor_set(x_440, 2, x_439); x_441 = lean_array_size(x_22); -x_442 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__4(x_441, x_16, x_22); +x_442 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__5(x_441, x_16, x_22); x_443 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__4; x_444 = l_Lean_mkSepArray(x_442, x_443); lean_dec(x_442); @@ -12723,7 +12815,7 @@ x_483 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__16; lean_inc(x_475); lean_inc(x_457); x_484 = l_Lean_Syntax_node2(x_457, x_483, x_475, x_482); -x_485 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_485 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_457); lean_ctor_set_tag(x_32, 2); lean_ctor_set(x_32, 1, x_485); @@ -12879,14 +12971,14 @@ if (lean_is_scalar(x_534)) { lean_ctor_set(x_536, 0, x_528); lean_ctor_set(x_536, 1, x_535); x_537 = l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__8; -x_538 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__5; +x_538 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__5; lean_inc(x_528); x_539 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_539, 0, x_528); lean_ctor_set(x_539, 1, x_537); lean_ctor_set(x_539, 2, x_538); x_540 = lean_array_size(x_22); -x_541 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__4(x_540, x_16, x_22); +x_541 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__5(x_540, x_16, x_22); x_542 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__4; x_543 = l_Lean_mkSepArray(x_541, x_542); lean_dec(x_541); @@ -13019,7 +13111,7 @@ x_582 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__16; lean_inc(x_574); lean_inc(x_556); x_583 = l_Lean_Syntax_node2(x_556, x_582, x_574, x_581); -x_584 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_584 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_556); x_585 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_585, 0, x_556); @@ -13250,14 +13342,14 @@ if (lean_is_scalar(x_657)) { lean_ctor_set(x_659, 0, x_651); lean_ctor_set(x_659, 1, x_658); x_660 = l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__8; -x_661 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__5; +x_661 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__5; lean_inc(x_651); x_662 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_662, 0, x_651); lean_ctor_set(x_662, 1, x_660); lean_ctor_set(x_662, 2, x_661); x_663 = lean_array_size(x_22); -x_664 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__4(x_663, x_16, x_22); +x_664 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__5(x_663, x_16, x_22); x_665 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__4; x_666 = l_Lean_mkSepArray(x_664, x_665); lean_dec(x_664); @@ -13390,7 +13482,7 @@ x_705 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__16; lean_inc(x_697); lean_inc(x_679); x_706 = l_Lean_Syntax_node2(x_679, x_705, x_697, x_704); -x_707 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_707 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_679); if (lean_is_scalar(x_634)) { x_708 = lean_alloc_ctor(2, 2, 0); @@ -13649,14 +13741,14 @@ if (lean_is_scalar(x_786)) { lean_ctor_set(x_788, 0, x_780); lean_ctor_set(x_788, 1, x_787); x_789 = l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__8; -x_790 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__5; +x_790 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__5; lean_inc(x_780); x_791 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_791, 0, x_780); lean_ctor_set(x_791, 1, x_789); lean_ctor_set(x_791, 2, x_790); x_792 = lean_array_size(x_750); -x_793 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__4(x_792, x_16, x_750); +x_793 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__5(x_792, x_16, x_750); x_794 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__4; x_795 = l_Lean_mkSepArray(x_793, x_794); lean_dec(x_793); @@ -13789,7 +13881,7 @@ x_834 = l_Lake_DSL_elabConfigDecl___lambda__2___closed__16; lean_inc(x_826); lean_inc(x_808); x_835 = l_Lean_Syntax_node2(x_808, x_834, x_826, x_833); -x_836 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6; +x_836 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6; lean_inc(x_808); if (lean_is_scalar(x_763)) { x_837 = lean_alloc_ctor(2, 2, 0); @@ -14139,6 +14231,15 @@ return x_76; } } } +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lake_DSL_elabConfigDecl___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_Lake_DSL_elabConfigDecl___spec__2(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; +} +} LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lake_DSL_elabConfigDecl___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { @@ -14149,7 +14250,7 @@ lean_dec(x_1); return x_6; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___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: { size_t x_9; size_t x_10; lean_object* x_11; @@ -14157,23 +14258,23 @@ x_9 = lean_unbox_usize(x_3); lean_dec(x_3); x_10 = lean_unbox_usize(x_4); lean_dec(x_4); -x_11 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2(x_1, x_2, x_9, x_10, x_5, x_6, x_7, x_8); +x_11 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3(x_1, x_2, x_9, x_10, x_5, x_6, x_7, x_8); lean_dec(x_7); lean_dec(x_2); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___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_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; -x_6 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4(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_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { size_t x_4; size_t x_5; lean_object* x_6; @@ -14181,44 +14282,44 @@ 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_Lake_DSL_elabConfigDecl___spec__4(x_4, x_5, x_3); +x_6 = l_Array_mapMUnsafe_map___at_Lake_DSL_elabConfigDecl___spec__5(x_4, x_5, x_3); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__6___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__7___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__6___lambda__1(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__7___lambda__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_Elab_Term_mkFreshIdent___at_Lake_DSL_elabConfigDecl___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshIdent___at_Lake_DSL_elabConfigDecl___spec__6___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_Elab_Term_mkFreshIdent___at_Lake_DSL_elabConfigDecl___spec__5(x_1, x_6, x_3, x_4, x_5); +x_7 = l_Lean_Elab_Term_mkFreshIdent___at_Lake_DSL_elabConfigDecl___spec__6(x_1, x_6, x_3, x_4, x_5); lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_mkIdentFromRef___at_Lake_DSL_elabConfigDecl___spec__7___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_mkIdentFromRef___at_Lake_DSL_elabConfigDecl___spec__8___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_mkIdentFromRef___at_Lake_DSL_elabConfigDecl___spec__7(x_1, x_6, x_3, x_4, x_5); +x_7 = l_Lean_mkIdentFromRef___at_Lake_DSL_elabConfigDecl___spec__8(x_1, x_6, x_3, x_4, x_5); lean_dec(x_4); lean_dec(x_3); return x_7; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___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_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { size_t x_11; size_t x_12; lean_object* x_13; @@ -14226,7 +14327,7 @@ x_11 = lean_unbox_usize(x_5); lean_dec(x_5); x_12 = lean_unbox_usize(x_6); lean_dec(x_6); -x_13 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__8(x_1, x_2, x_3, x_4, x_11, x_12, x_7, x_8, x_9, x_10); +x_13 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__9(x_1, x_2, x_3, x_4, x_11, x_12, x_7, x_8, x_9, x_10); lean_dec(x_9); lean_dec(x_4); lean_dec(x_3); @@ -14234,36 +14335,36 @@ lean_dec(x_2); return x_13; } } -LEAN_EXPORT lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___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_EXPORT lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; -x_7 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__9(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__10(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Array_sequenceMap_loop___at_Lake_DSL_elabConfigDecl___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Array_sequenceMap_loop___at_Lake_DSL_elabConfigDecl___spec__12___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; -x_6 = l_Array_sequenceMap_loop___at_Lake_DSL_elabConfigDecl___spec__11(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Array_sequenceMap_loop___at_Lake_DSL_elabConfigDecl___spec__12(x_1, x_2, x_3, x_4, x_5); lean_dec(x_1); return x_6; } } -LEAN_EXPORT lean_object* l_Array_sequenceMap___at_Lake_DSL_elabConfigDecl___spec__10___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_sequenceMap___at_Lake_DSL_elabConfigDecl___spec__11___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Array_sequenceMap___at_Lake_DSL_elabConfigDecl___spec__10(x_1, x_2); +x_3 = l_Array_sequenceMap___at_Lake_DSL_elabConfigDecl___spec__11(x_1, x_2); lean_dec(x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___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) { _start: { size_t x_10; size_t x_11; lean_object* x_12; @@ -14271,18 +14372,18 @@ x_10 = lean_unbox_usize(x_4); lean_dec(x_4); x_11 = lean_unbox_usize(x_5); lean_dec(x_5); -x_12 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__12(x_1, x_2, x_3, x_10, x_11, x_6, x_7, x_8, x_9); +x_12 = l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__13(x_1, x_2, x_3, x_10, x_11, x_6, x_7, x_8, x_9); lean_dec(x_8); lean_dec(x_3); lean_dec(x_2); return x_12; } } -LEAN_EXPORT lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___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_EXPORT lean_object* l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___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) { _start: { lean_object* x_7; -x_7 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__13(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__14(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_1); @@ -14725,50 +14826,50 @@ l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__7 = _init_l_Lake_DSL_expa lean_mark_persistent(l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__7); l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__8 = _init_l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__8(); lean_mark_persistent(l_Lake_DSL_expandOptSimpleBinder___lambda__1___closed__8); -l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__1); -l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__2 = _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__2(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__2); -l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__3 = _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__3(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__3); -l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__4 = _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__4(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__4); -l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__5 = _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__5(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__5); -l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__6 = _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__6(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__6); -l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__7 = _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__7(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__7); -l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__8 = _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__8(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__8); -l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__9 = _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__9(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__9); -l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__10 = _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__10(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__10); -l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__11 = _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__11(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__11); -l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__12 = _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__12(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__12); -l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__13 = _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__13(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__13); -l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__14 = _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__14(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__2___closed__14); -l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__1 = _init_l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__1(); -lean_mark_persistent(l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__1); -l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__2 = _init_l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__2(); -lean_mark_persistent(l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__2); -l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__3 = _init_l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__3(); -lean_mark_persistent(l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__3); -l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__4 = _init_l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__4(); -lean_mark_persistent(l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__4); -l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__5 = _init_l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__5(); -lean_mark_persistent(l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__5); -l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6 = _init_l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6(); -lean_mark_persistent(l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__3___closed__6); -l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__6___closed__1 = _init_l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__6___closed__1(); -lean_mark_persistent(l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__6___closed__1); -l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__6___closed__2 = _init_l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__6___closed__2(); -lean_mark_persistent(l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__6___closed__2); +l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__1(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__1); +l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__2 = _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__2(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__2); +l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__3 = _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__3(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__3); +l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__4 = _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__4(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__4); +l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__5 = _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__5(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__5); +l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__6 = _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__6(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__6); +l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__7 = _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__7(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__7); +l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__8 = _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__8(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__8); +l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__9 = _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__9(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__9); +l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__10 = _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__10(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__10); +l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__11 = _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__11(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__11); +l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__12 = _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__12(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__12); +l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__13 = _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__13(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__13); +l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__14 = _init_l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__14(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lake_DSL_elabConfigDecl___spec__3___closed__14); +l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__1 = _init_l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__1(); +lean_mark_persistent(l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__1); +l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__2 = _init_l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__2(); +lean_mark_persistent(l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__2); +l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__3 = _init_l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__3(); +lean_mark_persistent(l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__3); +l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__4 = _init_l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__4(); +lean_mark_persistent(l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__4); +l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__5 = _init_l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__5(); +lean_mark_persistent(l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__5); +l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6 = _init_l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6(); +lean_mark_persistent(l_Lean_RBNode_foldM___at_Lake_DSL_elabConfigDecl___spec__4___closed__6); +l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__7___closed__1 = _init_l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__7___closed__1(); +lean_mark_persistent(l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__7___closed__1); +l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__7___closed__2 = _init_l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__7___closed__2(); +lean_mark_persistent(l_Lean_Elab_Term_mkFreshBinderName___at_Lake_DSL_elabConfigDecl___spec__7___closed__2); l_Lake_DSL_elabConfigDecl___lambda__1___closed__1 = _init_l_Lake_DSL_elabConfigDecl___lambda__1___closed__1(); lean_mark_persistent(l_Lake_DSL_elabConfigDecl___lambda__1___closed__1); l_Lake_DSL_elabConfigDecl___lambda__1___closed__2 = _init_l_Lake_DSL_elabConfigDecl___lambda__1___closed__2(); diff --git a/stage0/stdlib/Lake/Load/Lean/Elab.c b/stage0/stdlib/Lake/Load/Lean/Elab.c index 450a4790aac7..70976656366a 100644 --- a/stage0/stdlib/Lake/Load/Lean/Elab.c +++ b/stage0/stdlib/Lake/Load/Lean/Elab.c @@ -133,6 +133,7 @@ lean_object* lean_st_mk_ref(lean_object*, lean_object*); lean_object* l_System_FilePath_fileName(lean_object*); static lean_object* l_Lake_importConfigFileCore_lakeExts___closed__34; static lean_object* l_Lake_importConfigFileCore_lakeExts___closed__23; +lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); static uint64_t l_Lake_importModulesUsingCache___closed__3; static lean_object* l_Lake_importConfigFileCore_lakeExts___closed__18; static lean_object* l_Lake_importConfigFileCore_lakeExts___closed__5; @@ -156,7 +157,6 @@ lean_object* lean_io_prim_handle_mk(lean_object*, uint8_t, lean_object*); LEAN_EXPORT lean_object* l_Lake_instFromJsonConfigTrace; lean_object* l_Lean_bignumFromJson_x3f(lean_object*); static lean_object* l___private_Lake_Load_Lean_Elab_0__Lake_fromJsonConfigTrace____x40_Lake_Load_Lean_Elab___hyg_1110____closed__11; -lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); static lean_object* l_Lake_configModuleName___closed__1; static lean_object* l_Lake_importConfigFileCore_lakeExts___closed__35; static lean_object* l_Lake_importConfigFileCore_lakeExts___closed__41; @@ -4635,7 +4635,7 @@ x_30 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_30, 0, x_10); lean_ctor_set(x_30, 1, x_29); x_31 = l___private_Lake_Load_Lean_Elab_0__Lake_toJsonConfigTrace____x40_Lake_Load_Lean_Elab___hyg_1030____closed__4; -x_32 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_30, x_31); +x_32 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_30, x_31); x_33 = l_Lean_Json_mkObj(x_32); return x_33; } diff --git a/stage0/stdlib/Lake/Util/Log.c b/stage0/stdlib/Lake/Util/Log.c index c3985d845651..a8b1217b01f9 100644 --- a/stage0/stdlib/Lake/Util/Log.c +++ b/stage0/stdlib/Lake/Util/Log.c @@ -24,6 +24,7 @@ LEAN_EXPORT lean_object* l_Lake_LogT_run___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_MonadLogT_adaptMethods___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lake_Util_Log_0__Lake_reprVerbosity____x40_Lake_Util_Log___hyg_9____closed__2; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lake_Log_toString___spec__1(lean_object*, size_t, size_t, lean_object*); +lean_object* l_Array_take___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_LogLevel_ofMessageSeverity___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lake_logError___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_Log_isEmpty___boxed(lean_object*); @@ -113,6 +114,7 @@ LEAN_EXPORT lean_object* l_Lake_logWarning(lean_object*); LEAN_EXPORT lean_object* l_Lake_Log_replay___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_MonadLog_ofMonadState(lean_object*); LEAN_EXPORT lean_object* l_Lake_logVerbose___rarg(lean_object*, lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); static lean_object* l_Lake_getLogPos___rarg___closed__1; static lean_object* l_Lake_LogLevel_ofString_x3f___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lake_instFromJsonLog___spec__1___boxed(lean_object*, lean_object*, lean_object*); @@ -328,7 +330,6 @@ static lean_object* l_Lake_LogLevel_ofString_x3f___closed__6; LEAN_EXPORT lean_object* l_Lake_ELogT_takeAndRun___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lake_Util_Log_0__Lake_reprLogLevel____x40_Lake_Util_Log___hyg_505____closed__2; lean_object* l_Substring_takeWhileAux___at_Substring_trimLeft___spec__1(lean_object*, lean_object*, lean_object*); -lean_object* l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_Log_takeFrom___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_ELogT_replayLog_x3f___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_instToStringLogEntry(lean_object*); @@ -394,7 +395,6 @@ lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_extractLog___rarg___lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_instToStringLogLevel; LEAN_EXPORT lean_object* l_Lake_instMaxVerbosity___boxed(lean_object*, lean_object*); -lean_object* l_Array_shrink___rarg(lean_object*, lean_object*); static lean_object* l___private_Lake_Util_Log_0__Lake_fromJsonLogEntry____x40_Lake_Util_Log___hyg_1450____closed__11; LEAN_EXPORT lean_object* l_Lake_ELogT_replayLog_x3f___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lake_Util_Log_0__Lake_fromJsonLogLevel____x40_Lake_Util_Log___hyg_917____closed__3; @@ -3128,7 +3128,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_7); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lake_Util_Log_0__Lake_fromJsonLogLevel____x40_Lake_Util_Log___hyg_917____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -5149,7 +5149,7 @@ LEAN_EXPORT lean_object* l_Lake_Log_dropFrom(lean_object* x_1, lean_object* x_2) _start: { lean_object* x_3; -x_3 = l_Array_shrink___rarg(x_1, x_2); +x_3 = l_Array_take___rarg(x_1, x_2); return x_3; } } @@ -5186,7 +5186,7 @@ LEAN_EXPORT lean_object* l_Lake_Log_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; lean_inc(x_1); -x_3 = l_Array_shrink___rarg(x_1, x_2); +x_3 = l_Array_take___rarg(x_1, x_2); x_4 = lean_array_get_size(x_1); x_5 = l_Array_extract___rarg(x_1, x_2, x_4); lean_dec(x_4); @@ -5898,7 +5898,7 @@ x_3 = lean_array_get_size(x_2); lean_inc(x_1); x_4 = l_Array_extract___rarg(x_2, x_1, x_3); lean_dec(x_3); -x_5 = l_Array_shrink___rarg(x_2, x_1); +x_5 = l_Array_take___rarg(x_2, x_1); lean_dec(x_1); x_6 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_6, 0, x_4); @@ -5931,7 +5931,7 @@ LEAN_EXPORT lean_object* l_Lake_dropLogFrom___rarg___lambda__1(lean_object* x_1, _start: { lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_3 = l_Array_shrink___rarg(x_2, x_1); +x_3 = l_Array_take___rarg(x_2, x_1); x_4 = lean_box(0); x_5 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_5, 0, x_4); @@ -7528,7 +7528,7 @@ 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; x_7 = lean_ctor_get(x_4, 0); x_8 = lean_ctor_get(x_4, 1); -x_9 = l_Array_shrink___rarg(x_8, x_7); +x_9 = l_Array_take___rarg(x_8, x_7); lean_dec(x_7); x_10 = lean_box(0); lean_ctor_set_tag(x_4, 0); @@ -7550,7 +7550,7 @@ x_15 = lean_ctor_get(x_4, 1); lean_inc(x_15); lean_inc(x_14); lean_dec(x_4); -x_16 = l_Array_shrink___rarg(x_15, x_14); +x_16 = l_Array_take___rarg(x_15, x_14); lean_dec(x_14); x_17 = lean_box(0); x_18 = lean_alloc_ctor(0, 2, 0); @@ -7848,7 +7848,7 @@ x_20 = lean_array_get_size(x_17); lean_inc(x_16); x_21 = l_Array_extract___rarg(x_17, x_16, x_20); lean_dec(x_20); -x_22 = l_Array_shrink___rarg(x_17, x_16); +x_22 = l_Array_take___rarg(x_17, x_16); lean_dec(x_16); lean_ctor_set_tag(x_4, 0); lean_ctor_set(x_4, 1, x_22); @@ -7877,7 +7877,7 @@ x_30 = lean_array_get_size(x_27); lean_inc(x_26); x_31 = l_Array_extract___rarg(x_27, x_26, x_30); lean_dec(x_30); -x_32 = l_Array_shrink___rarg(x_27, x_26); +x_32 = l_Array_take___rarg(x_27, x_26); lean_dec(x_26); x_33 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_33, 0, x_31); diff --git a/stage0/stdlib/Lean.c b/stage0/stdlib/Lean.c index 3688e5cf6c25..eee8e4226bfe 100644 --- a/stage0/stdlib/Lean.c +++ b/stage0/stdlib/Lean.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Lean -// Imports: Init Lean.Data Lean.Compiler Lean.Environment Lean.Modifiers Lean.ProjFns Lean.Runtime Lean.ResolveName Lean.Attributes Lean.Parser Lean.ReducibilityAttrs Lean.Elab Lean.Class Lean.LocalContext Lean.MetavarContext Lean.AuxRecursor Lean.Meta Lean.Util Lean.Structure Lean.PrettyPrinter Lean.CoreM Lean.ReservedNameAction Lean.InternalExceptionId Lean.Server Lean.ScopedEnvExtension Lean.DocString Lean.DeclarationRange Lean.LazyInitExtension Lean.LoadDynlib Lean.Widget Lean.Log Lean.Linter Lean.SubExpr Lean.LabelAttribute Lean.AddDecl Lean.Replay +// Imports: Init Lean.Data Lean.Compiler Lean.Environment Lean.Modifiers Lean.ProjFns Lean.Runtime Lean.ResolveName Lean.Attributes Lean.Parser Lean.ReducibilityAttrs Lean.Elab Lean.Class Lean.LocalContext Lean.MetavarContext Lean.AuxRecursor Lean.Meta Lean.Util Lean.Structure Lean.PrettyPrinter Lean.CoreM Lean.ReservedNameAction Lean.InternalExceptionId Lean.Server Lean.ScopedEnvExtension Lean.DocString Lean.DeclarationRange Lean.LoadDynlib Lean.Widget Lean.Log Lean.Linter Lean.SubExpr Lean.LabelAttribute Lean.AddDecl Lean.Replay #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -40,7 +40,6 @@ lean_object* initialize_Lean_Server(uint8_t builtin, lean_object*); lean_object* initialize_Lean_ScopedEnvExtension(uint8_t builtin, lean_object*); lean_object* initialize_Lean_DocString(uint8_t builtin, lean_object*); lean_object* initialize_Lean_DeclarationRange(uint8_t builtin, lean_object*); -lean_object* initialize_Lean_LazyInitExtension(uint8_t builtin, lean_object*); lean_object* initialize_Lean_LoadDynlib(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Widget(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Log(uint8_t builtin, lean_object*); @@ -135,9 +134,6 @@ lean_dec_ref(res); res = initialize_Lean_DeclarationRange(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -res = initialize_Lean_LazyInitExtension(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Lean_LoadDynlib(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Lean/Compiler/IR/Basic.c b/stage0/stdlib/Lean/Compiler/IR/Basic.c index b4a4d956d7d3..c1839357c49d 100644 --- a/stage0/stdlib/Lean/Compiler/IR/Basic.c +++ b/stage0/stdlib/Lean/Compiler/IR/Basic.c @@ -5244,7 +5244,7 @@ x_13 = l_Lean_IR_reshapeAux___closed__2; x_14 = lean_string_append(x_12, x_13); x_15 = l_Lean_IR_reshapeAux___closed__3; x_16 = l_Lean_IR_reshapeAux___closed__4; -x_17 = lean_unsigned_to_nat(220u); +x_17 = lean_unsigned_to_nat(258u); x_18 = lean_unsigned_to_nat(4u); x_19 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_15, x_16, x_17, x_18, x_14); lean_dec(x_14); diff --git a/stage0/stdlib/Lean/Compiler/IR/ElimDeadBranches.c b/stage0/stdlib/Lean/Compiler/IR/ElimDeadBranches.c index e2c938382024..aa583e4f6835 100644 --- a/stage0/stdlib/Lean/Compiler/IR/ElimDeadBranches.c +++ b/stage0/stdlib/Lean/Compiler/IR/ElimDeadBranches.c @@ -161,13 +161,14 @@ LEAN_EXPORT uint8_t l_Lean_IR_UnreachableBranches_Value_toFormat___lambda__1(lea static lean_object* l_Lean_IR_UnreachableBranches_interpFnBody___closed__4; static lean_object* l_List_mapTR_loop___at_Lean_IR_UnreachableBranches_Value_toFormat___spec__1___closed__2; lean_object* l_Lean_IR_LocalContext_getJPParams(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_elimDeadBranches___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_elimDeadBranches___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_repr___at___private_Lean_Compiler_IR_ElimDeadBranches_0__Lean_IR_UnreachableBranches_reprValue____x40_Lean_Compiler_IR_ElimDeadBranches___hyg_42____spec__4___closed__10; static lean_object* l___private_Lean_Compiler_IR_ElimDeadBranches_0__Lean_IR_UnreachableBranches_reprValue____x40_Lean_Compiler_IR_ElimDeadBranches___hyg_42____closed__4; LEAN_EXPORT lean_object* l_Lean_IR_formatArray___at_Lean_IR_UnreachableBranches_Value_format___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_IR_UnreachableBranches_inferStep(lean_object*, lean_object*); static lean_object* l_List_repr___at___private_Lean_Compiler_IR_ElimDeadBranches_0__Lean_IR_UnreachableBranches_reprValue____x40_Lean_Compiler_IR_ElimDeadBranches___hyg_42____spec__4___closed__7; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_UnreachableBranches_Value_truncate_go___spec__10(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_elimDeadBranches___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_modifyAux___at_Lean_IR_UnreachableBranches_updateCurrFnSummary___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_IR_UnreachableBranches_Value_toFormat(lean_object*); lean_object* l_Lean_IR_Decl_name(lean_object*); @@ -328,7 +329,6 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_UnreachableBranches static lean_object* l___private_Lean_Compiler_IR_ElimDeadBranches_0__Lean_IR_UnreachableBranches_reprValue____x40_Lean_Compiler_IR_ElimDeadBranches___hyg_42____closed__12; static lean_object* l_Lean_IR_UnreachableBranches_Value_addChoice___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_UnreachableBranches_Value_truncate_go___spec__5(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_elimDeadBranches___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_uget(lean_object*, size_t); size_t lean_array_size(lean_object*); LEAN_EXPORT lean_object* l_Std_Format_joinSep___at___private_Lean_Compiler_IR_ElimDeadBranches_0__Lean_IR_UnreachableBranches_reprValue____x40_Lean_Compiler_IR_ElimDeadBranches___hyg_42____spec__2(lean_object*, lean_object*); @@ -10382,7 +10382,7 @@ return x_6; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_elimDeadBranches___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_elimDeadBranches___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; uint8_t x_9; @@ -10483,7 +10483,7 @@ lean_inc(x_9); x_22 = l_Nat_foldTR_loop___at_Lean_IR_elimDeadBranches___spec__1(x_1, x_9, x_20, x_9, x_9, x_5); lean_ctor_set(x_3, 0, x_22); x_23 = lean_mk_empty_array_with_capacity(x_9); -x_24 = l_Array_mapIdxM_map___at_Lean_IR_elimDeadBranches___spec__2(x_1, x_21, x_1, x_9, x_13, lean_box(0), x_23); +x_24 = l_Array_mapFinIdxM_map___at_Lean_IR_elimDeadBranches___spec__2(x_1, x_21, x_1, x_9, x_13, lean_box(0), x_23); lean_dec(x_21); lean_dec(x_1); lean_ctor_set(x_16, 1, x_3); @@ -10505,7 +10505,7 @@ lean_inc(x_9); x_28 = l_Nat_foldTR_loop___at_Lean_IR_elimDeadBranches___spec__1(x_1, x_9, x_26, x_9, x_9, x_5); lean_ctor_set(x_3, 0, x_28); x_29 = lean_mk_empty_array_with_capacity(x_9); -x_30 = l_Array_mapIdxM_map___at_Lean_IR_elimDeadBranches___spec__2(x_1, x_27, x_1, x_9, x_13, lean_box(0), x_29); +x_30 = l_Array_mapFinIdxM_map___at_Lean_IR_elimDeadBranches___spec__2(x_1, x_27, x_1, x_9, x_13, lean_box(0), x_29); lean_dec(x_27); lean_dec(x_1); x_31 = lean_alloc_ctor(0, 2, 0); @@ -10564,7 +10564,7 @@ x_50 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_50, 0, x_49); lean_ctor_set(x_50, 1, x_33); x_51 = lean_mk_empty_array_with_capacity(x_37); -x_52 = l_Array_mapIdxM_map___at_Lean_IR_elimDeadBranches___spec__2(x_1, x_48, x_1, x_37, x_41, lean_box(0), x_51); +x_52 = l_Array_mapFinIdxM_map___at_Lean_IR_elimDeadBranches___spec__2(x_1, x_48, x_1, x_37, x_41, lean_box(0), x_51); lean_dec(x_48); lean_dec(x_1); if (lean_is_scalar(x_46)) { @@ -10589,11 +10589,11 @@ lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_elimDeadBranches___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_elimDeadBranches___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; -x_8 = l_Array_mapIdxM_map___at_Lean_IR_elimDeadBranches___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Array_mapFinIdxM_map___at_Lean_IR_elimDeadBranches___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); diff --git a/stage0/stdlib/Lean/Compiler/IR/PushProj.c b/stage0/stdlib/Lean/Compiler/IR/PushProj.c index 45973f1db7ed..a8d4d8f238f7 100644 --- a/stage0/stdlib/Lean/Compiler/IR/PushProj.c +++ b/stage0/stdlib/Lean/Compiler/IR/PushProj.c @@ -13,36 +13,38 @@ #ifdef __cplusplus extern "C" { #endif -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__5___at_Lean_IR_pushProjs___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__9___at_Lean_IR_pushProjs___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__5___at_Lean_IR_pushProjs___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_pushProjs___spec__7___at_Lean_IR_pushProjs___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__9___at_Lean_IR_pushProjs___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__1___at_Lean_IR_pushProjs___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_pushProjs___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_IR_instInhabitedFnBody; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_pushProjs___spec__11___at_Lean_IR_pushProjs___spec__12(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_pushProjs___spec__11(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_pushProjs___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_pushProjs___spec__11___at_Lean_IR_pushProjs___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__5___at_Lean_IR_pushProjs___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_IR_FnBody_flatten(lean_object*); lean_object* l_Lean_IR_FnBody_freeIndices(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__9___at_Lean_IR_pushProjs___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_reverse___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__1___at_Lean_IR_pushProjs___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_FnBody_pushProj___spec__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_IR_FnBody_pushProj___closed__1; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_IR_Decl_pushProj(lean_object*); lean_object* lean_array_pop(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_IR_pushProjs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_FnBody_pushProj___spec__3(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_FnBody_pushProj___spec__2(size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__1___at_Lean_IR_pushProjs___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_IR_instInhabitedIndexSet; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__1___at_Lean_IR_pushProjs___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_pushProjs___spec__3(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_IR_FnBody_pushProj(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_FnBody_pushProj___spec__1(size_t, size_t, lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); @@ -50,8 +52,8 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_pushProjs___spec__7 LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_pushProjs___spec__3___at_Lean_IR_pushProjs___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_IR_FnBody_setBody(lean_object*, lean_object*); lean_object* l_Lean_IR_Decl_updateBody_x21(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__9___at_Lean_IR_pushProjs___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_FnBody_pushProj___spec__3___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_IR_AltCore_body(lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); @@ -61,24 +63,22 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_pushProjs___spec__7 lean_object* lean_array_mk(lean_object*); size_t lean_usize_add(size_t, size_t); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_pushProjs___spec__3___at_Lean_IR_pushProjs___spec__4(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_IR_mkIndexSet(lean_object*); lean_object* lean_array_uget(lean_object*, size_t); size_t lean_array_size(lean_object*); lean_object* l_Lean_IR_FnBody_collectFreeIndices(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__5___at_Lean_IR_pushProjs___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_RBNode_findCore___at_Lean_IR_UniqueIds_checkId___spec__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); lean_object* l_Lean_IR_reshape(lean_object*, lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); lean_object* l_Lean_IR_Decl_normalizeIds(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_FnBody_pushProj___spec__2___boxed(lean_object*, lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_uset(lean_object*, size_t, lean_object*); lean_object* lean_array_get(lean_object*, lean_object*, lean_object*); uint8_t l_Array_isEmpty___rarg(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; uint8_t x_12; @@ -262,7 +262,7 @@ return x_10; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__1___at_Lean_IR_pushProjs___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__1___at_Lean_IR_pushProjs___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { lean_object* x_10; uint8_t x_11; @@ -528,7 +528,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; uint8_t x_12; @@ -712,7 +712,7 @@ return x_10; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__5___at_Lean_IR_pushProjs___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__5___at_Lean_IR_pushProjs___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { lean_object* x_10; uint8_t x_11; @@ -978,7 +978,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; uint8_t x_12; @@ -1162,7 +1162,7 @@ return x_10; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__9___at_Lean_IR_pushProjs___spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__9___at_Lean_IR_pushProjs___spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { lean_object* x_10; uint8_t x_11; @@ -1510,7 +1510,7 @@ x_27 = lean_array_get_size(x_2); x_28 = lean_mk_empty_array_with_capacity(x_27); x_29 = lean_unsigned_to_nat(0u); lean_inc(x_8); -x_30 = l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__1___at_Lean_IR_pushProjs___spec__2(x_2, x_3, x_8, x_25, x_2, x_27, x_29, lean_box(0), x_28); +x_30 = l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__1___at_Lean_IR_pushProjs___spec__2(x_2, x_3, x_8, x_25, x_2, x_27, x_29, lean_box(0), x_28); lean_dec(x_2); x_31 = lean_array_size(x_3); x_32 = 0; @@ -1549,7 +1549,7 @@ x_40 = lean_array_get_size(x_2); x_41 = lean_mk_empty_array_with_capacity(x_40); x_42 = lean_unsigned_to_nat(0u); lean_inc(x_8); -x_43 = l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__5___at_Lean_IR_pushProjs___spec__6(x_2, x_3, x_8, x_38, x_2, x_40, x_42, lean_box(0), x_41); +x_43 = l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__5___at_Lean_IR_pushProjs___spec__6(x_2, x_3, x_8, x_38, x_2, x_40, x_42, lean_box(0), x_41); lean_dec(x_2); x_44 = lean_array_size(x_3); x_45 = 0; @@ -1588,7 +1588,7 @@ x_53 = lean_array_get_size(x_2); x_54 = lean_mk_empty_array_with_capacity(x_53); x_55 = lean_unsigned_to_nat(0u); lean_inc(x_8); -x_56 = l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__9___at_Lean_IR_pushProjs___spec__10(x_2, x_3, x_8, x_51, x_2, x_53, x_55, lean_box(0), x_54); +x_56 = l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__9___at_Lean_IR_pushProjs___spec__10(x_2, x_3, x_8, x_51, x_2, x_53, x_55, lean_box(0), x_54); lean_dec(x_2); x_57 = lean_array_size(x_3); x_58 = 0; @@ -1831,11 +1831,11 @@ return x_117; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; -x_11 = l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); @@ -1844,11 +1844,11 @@ lean_dec(x_1); return x_11; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__1___at_Lean_IR_pushProjs___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__1___at_Lean_IR_pushProjs___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { lean_object* x_10; -x_10 = l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__1___at_Lean_IR_pushProjs___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_10 = l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__1___at_Lean_IR_pushProjs___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); @@ -1883,11 +1883,11 @@ lean_dec(x_2); return x_8; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; -x_11 = l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); @@ -1896,11 +1896,11 @@ lean_dec(x_1); return x_11; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__5___at_Lean_IR_pushProjs___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__5___at_Lean_IR_pushProjs___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { lean_object* x_10; -x_10 = l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__5___at_Lean_IR_pushProjs___spec__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_10 = l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__5___at_Lean_IR_pushProjs___spec__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); @@ -1935,11 +1935,11 @@ lean_dec(x_2); return x_8; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; -x_11 = l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__9(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__9(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); @@ -1948,11 +1948,11 @@ lean_dec(x_1); return x_11; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__9___at_Lean_IR_pushProjs___spec__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__9___at_Lean_IR_pushProjs___spec__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { lean_object* x_10; -x_10 = l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__9___at_Lean_IR_pushProjs___spec__10(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_10 = l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__9___at_Lean_IR_pushProjs___spec__10(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); diff --git a/stage0/stdlib/Lean/Compiler/LCNF/ElimDeadBranches.c b/stage0/stdlib/Lean/Compiler/LCNF/ElimDeadBranches.c index 42308d51761d..97bc8fdbe112 100644 --- a/stage0/stdlib/Lean/Compiler/LCNF/ElimDeadBranches.c +++ b/stage0/stdlib/Lean/Compiler/LCNF/ElimDeadBranches.c @@ -122,6 +122,7 @@ lean_object* l_Nat_nextPowerOfTwo_go(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Compiler_LCNF_UnreachableBranches_instReprValue___closed__1; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_UnreachableBranches_elimDead_go___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Environment_addExtraName(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Compiler_LCNF_Decl_elimDeadBranches___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Prod_repr___at_Lean_Compiler_LCNF_UnreachableBranches_elimDead___spec__4___boxed(lean_object*, lean_object*); static lean_object* l_panic___at_Lean_Compiler_LCNF_UnreachableBranches_Value_getLiteral_go___spec__1___closed__5; uint8_t l___private_Lean_Util_Trace_0__Lean_checkTraceOption(lean_object*, lean_object*, lean_object*); @@ -130,7 +131,6 @@ static lean_object* l_List_repr___at___private_Lean_Compiler_LCNF_ElimDeadBranch uint8_t l_List_any___rarg(lean_object*, lean_object*); uint8_t lean_string_dec_eq(lean_object*, lean_object*); static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_ElimDeadBranches___hyg_6212____closed__8; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Compiler_LCNF_Decl_elimDeadBranches___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_Compiler_LCNF_UnreachableBranches_getFunctionSummary_x3f___spec__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Compiler_LCNF_UnreachableBranches_Value_beq___lambda__1(lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Compiler_LCNF_UnreachableBranches_inferMain___spec__1___closed__2; @@ -221,13 +221,13 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Compiler_LCNF_Unreacha static lean_object* l_Lean_Compiler_LCNF_UnreachableBranches_initFn____x40_Lean_Compiler_LCNF_ElimDeadBranches___hyg_1931____closed__3; static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_ElimDeadBranches___hyg_6212____closed__1; lean_object* l_Lean_MessageData_ofFormat(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Compiler_LCNF_Decl_elimDeadBranches___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Compiler_LCNF_UnreachableBranches_initFn____x40_Lean_Compiler_LCNF_ElimDeadBranches___hyg_1931____closed__9; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_UnreachableBranches_instInhabitedValue; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Compiler_LCNF_UnreachableBranches_interpCode___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_outOfBounds___rarg(lean_object*); LEAN_EXPORT lean_object* l_repr___at_Lean_Compiler_LCNF_UnreachableBranches_elimDead___spec__3(lean_object*); static lean_object* l_Lean_Compiler_LCNF_UnreachableBranches_Value_ofNat_goSmall___closed__2; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Compiler_LCNF_Decl_elimDeadBranches___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Compiler_LCNF_UnreachableBranches_Value_truncate_go___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_ElimDeadBranches___hyg_6212____closed__15; @@ -18316,7 +18316,7 @@ return x_6; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Compiler_LCNF_Decl_elimDeadBranches___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Compiler_LCNF_Decl_elimDeadBranches___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; uint8_t x_14; @@ -18575,7 +18575,7 @@ x_35 = lean_ctor_get(x_34, 1); lean_inc(x_35); lean_dec(x_34); x_36 = lean_mk_empty_array_with_capacity(x_10); -x_37 = l_Array_mapIdxM_map___at_Lean_Compiler_LCNF_Decl_elimDeadBranches___spec__3(x_1, x_25, x_1, x_10, x_13, lean_box(0), x_36, x_2, x_3, x_4, x_5, x_35); +x_37 = l_Array_mapFinIdxM_map___at_Lean_Compiler_LCNF_Decl_elimDeadBranches___spec__3(x_1, x_25, x_1, x_10, x_13, lean_box(0), x_36, x_2, x_3, x_4, x_5, x_35); lean_dec(x_25); lean_dec(x_1); return x_37; @@ -18612,7 +18612,7 @@ x_48 = lean_ctor_get(x_47, 1); lean_inc(x_48); lean_dec(x_47); x_49 = lean_mk_empty_array_with_capacity(x_10); -x_50 = l_Array_mapIdxM_map___at_Lean_Compiler_LCNF_Decl_elimDeadBranches___spec__3(x_1, x_25, x_1, x_10, x_13, lean_box(0), x_49, x_2, x_3, x_4, x_5, x_48); +x_50 = l_Array_mapFinIdxM_map___at_Lean_Compiler_LCNF_Decl_elimDeadBranches___spec__3(x_1, x_25, x_1, x_10, x_13, lean_box(0), x_49, x_2, x_3, x_4, x_5, x_48); lean_dec(x_25); lean_dec(x_1); return x_50; @@ -18670,11 +18670,11 @@ lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Compiler_LCNF_Decl_elimDeadBranches___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Compiler_LCNF_Decl_elimDeadBranches___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; -x_13 = l_Array_mapIdxM_map___at_Lean_Compiler_LCNF_Decl_elimDeadBranches___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_13 = l_Array_mapFinIdxM_map___at_Lean_Compiler_LCNF_Decl_elimDeadBranches___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); diff --git a/stage0/stdlib/Lean/Compiler/LCNF/PullLetDecls.c b/stage0/stdlib/Lean/Compiler/LCNF/PullLetDecls.c index ba74b28216d0..72470ff92ccf 100644 --- a/stage0/stdlib/Lean/Compiler/LCNF/PullLetDecls.c +++ b/stage0/stdlib/Lean/Compiler/LCNF/PullLetDecls.c @@ -15,6 +15,7 @@ extern "C" { #endif LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_PullLetDecls_attachToPull___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Decl_pullLetDecls___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_take___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Compiler_LCNF_pullInstances___closed__2; LEAN_EXPORT lean_object* l___private_Init_Data_Array_BasicAux_0__mapMonoMImp_go___at_Lean_Compiler_LCNF_PullLetDecls_pullDecls___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_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_PullLetDecls___hyg_1316____closed__5; @@ -92,7 +93,6 @@ static lean_object* l_Lean_Compiler_LCNF_pullInstances___closed__3; lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_Decl_pullInstances___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Compiler_LCNF_PullLetDecls_withParams___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Array_shrink___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_PullLetDecls_pullDecls___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_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_PullLetDecls___hyg_1316____closed__16; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_PullLetDecls_attachToPull(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -490,7 +490,7 @@ lean_inc(x_27); x_28 = lean_ctor_get(x_26, 1); lean_inc(x_28); lean_dec(x_26); -x_29 = l_Array_shrink___rarg(x_27, x_12); +x_29 = l_Array_take___rarg(x_27, x_12); lean_dec(x_12); x_30 = l_Array_append___rarg(x_29, x_25); lean_dec(x_25); @@ -586,7 +586,7 @@ lean_inc(x_55); x_56 = lean_ctor_get(x_54, 1); lean_inc(x_56); lean_dec(x_54); -x_57 = l_Array_shrink___rarg(x_55, x_12); +x_57 = l_Array_take___rarg(x_55, x_12); lean_dec(x_12); x_58 = l_Array_append___rarg(x_57, x_53); lean_dec(x_53); diff --git a/stage0/stdlib/Lean/Data/Lsp/Basic.c b/stage0/stdlib/Lean/Data/Lsp/Basic.c index 3743cc64aad2..32a9dea6abde 100644 --- a/stage0/stdlib/Lean/Data/Lsp/Basic.c +++ b/stage0/stdlib/Lean/Data/Lsp/Basic.c @@ -392,6 +392,7 @@ static lean_object* l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonLocation LEAN_EXPORT lean_object* l_Lean_Lsp_instToStringPosition(lean_object*); static lean_object* l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonDeleteFile____x40_Lean_Data_Lsp_Basic___hyg_3950____closed__3; LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonCreateFile; +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_ins___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonWorkspaceEdit____x40_Lean_Data_Lsp_Basic___hyg_4439____spec__3(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_CreateFile_toJsonOptions____x40_Lean_Data_Lsp_Basic___hyg_3022____closed__2; LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonLocationLink; @@ -452,7 +453,6 @@ LEAN_EXPORT lean_object* l_Lean_RBNode_foldM___at___private_Lean_Data_Lsp_Basic_ static lean_object* l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonWorkspaceEdit____x40_Lean_Data_Lsp_Basic___hyg_4439____closed__7; static lean_object* l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonStaticRegistrationOptions____x40_Lean_Data_Lsp_Basic___hyg_5746____closed__6; static lean_object* l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonLocationLink____x40_Lean_Data_Lsp_Basic___hyg_1410____closed__7; -LEAN_EXPORT lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonSnippetString____x40_Lean_Data_Lsp_Basic___hyg_1878____closed__6; LEAN_EXPORT lean_object* l_Lean_RBNode_ins___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonWorkspaceEdit____x40_Lean_Data_Lsp_Basic___hyg_4439____spec__18(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonDeleteFile____x40_Lean_Data_Lsp_Basic___hyg_3904_(lean_object*); @@ -932,7 +932,7 @@ x_1 = l_Lean_Lsp_instBEqCancelParams___closed__1; return x_1; } } -LEAN_EXPORT lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -1034,7 +1034,7 @@ x_7 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_7, 0, x_6); lean_ctor_set(x_7, 1, x_2); x_8 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -1057,7 +1057,7 @@ x_16 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_16, 0, x_15); lean_ctor_set(x_16, 1, x_2); x_17 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_18 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_16, x_17); +x_18 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_16, x_17); x_19 = l_Lean_Json_mkObj(x_18); return x_19; } @@ -1081,7 +1081,7 @@ x_24 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_24, 0, x_23); lean_ctor_set(x_24, 1, x_2); x_25 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_26 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_24, x_25); +x_26 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_24, x_25); x_27 = l_Lean_Json_mkObj(x_26); return x_27; } @@ -1104,7 +1104,7 @@ x_33 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_33, 0, x_32); lean_ctor_set(x_33, 1, x_2); x_34 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_35 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_33, x_34); +x_35 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_33, x_34); x_36 = l_Lean_Json_mkObj(x_35); return x_36; } @@ -1114,7 +1114,7 @@ return x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; x_37 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__5; x_38 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_39 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_37, x_38); +x_39 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_37, x_38); x_40 = l_Lean_Json_mkObj(x_39); return x_40; } @@ -1591,7 +1591,7 @@ x_16 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_16, 0, x_8); lean_ctor_set(x_16, 1, x_15); x_17 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_18 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_16, x_17); +x_18 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_16, x_17); x_19 = l_Lean_Json_mkObj(x_18); return x_19; } @@ -2093,7 +2093,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_7); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -2581,7 +2581,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_8); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -2618,7 +2618,7 @@ x_30 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_30, 0, x_24); lean_ctor_set(x_30, 1, x_29); x_31 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_32 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_30, x_31); +x_32 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_30, x_31); x_33 = l_Lean_Json_mkObj(x_32); return x_33; } @@ -3104,7 +3104,7 @@ x_24 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_24, 0, x_4); lean_ctor_set(x_24, 1, x_23); x_25 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_26 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_24, x_25); +x_26 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_24, x_25); x_27 = l_Lean_Json_mkObj(x_26); return x_27; } @@ -3878,7 +3878,7 @@ x_18 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_18, 0, x_9); lean_ctor_set(x_18, 1, x_17); x_19 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_20 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_18, x_19); +x_20 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_18, x_19); x_21 = l_Lean_Json_mkObj(x_20); return x_21; } @@ -4462,7 +4462,7 @@ x_7 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_7, 0, x_6); lean_ctor_set(x_7, 1, x_5); x_8 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -4782,7 +4782,7 @@ x_22 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_22, 0, x_7); lean_ctor_set(x_22, 1, x_21); x_23 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_24 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_22, x_23); +x_24 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_22, x_23); x_25 = l_Lean_Json_mkObj(x_24); return x_25; } @@ -5818,7 +5818,7 @@ x_7 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_7, 0, x_6); lean_ctor_set(x_7, 1, x_5); x_8 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -6057,7 +6057,7 @@ x_12 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_12, 0, x_8); lean_ctor_set(x_12, 1, x_11); x_13 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_14 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); +x_14 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); x_15 = l_Lean_Json_mkObj(x_14); return x_15; } @@ -6088,7 +6088,7 @@ x_26 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_26, 0, x_22); lean_ctor_set(x_26, 1, x_25); x_27 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_28 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_26, x_27); +x_28 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_26, x_27); x_29 = l_Lean_Json_mkObj(x_28); return x_29; } @@ -6571,7 +6571,7 @@ x_17 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_17, 0, x_7); lean_ctor_set(x_17, 1, x_16); x_18 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_19 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_17, x_18); +x_19 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_17, x_18); x_20 = l_Lean_Json_mkObj(x_19); return x_20; } @@ -7009,7 +7009,7 @@ x_18 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_18, 0, x_9); lean_ctor_set(x_18, 1, x_17); x_19 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_20 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_18, x_19); +x_20 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_18, x_19); x_21 = l_Lean_Json_mkObj(x_20); return x_21; } @@ -7435,7 +7435,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_8); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -7772,7 +7772,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_8); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -8123,7 +8123,7 @@ x_16 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_16, 0, x_9); lean_ctor_set(x_16, 1, x_15); x_17 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_18 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_16, x_17); +x_18 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_16, x_17); x_19 = l_Lean_Json_mkObj(x_18); return x_19; } @@ -8682,7 +8682,7 @@ x_22 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_22, 0, x_10); lean_ctor_set(x_22, 1, x_21); x_23 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_24 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_22, x_23); +x_24 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_22, x_23); x_25 = l_Lean_Json_mkObj(x_24); return x_25; } @@ -9134,7 +9134,7 @@ x_16 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_16, 0, x_9); lean_ctor_set(x_16, 1, x_15); x_17 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_18 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_16, x_17); +x_18 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_16, x_17); x_19 = l_Lean_Json_mkObj(x_18); return x_19; } @@ -10502,7 +10502,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_4); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -20468,7 +20468,7 @@ x_12 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_12, 0, x_4); lean_ctor_set(x_12, 1, x_11); x_13 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_14 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); +x_14 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); x_15 = l_Lean_Json_mkObj(x_14); return x_15; } @@ -20837,7 +20837,7 @@ x_27 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_27, 0, x_10); lean_ctor_set(x_27, 1, x_26); x_28 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_29 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_27, x_28); +x_29 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_27, x_28); x_30 = l_Lean_Json_mkObj(x_29); return x_30; } @@ -21289,7 +21289,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_7); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -21639,7 +21639,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_4); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -22218,7 +22218,7 @@ x_5 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_5, 0, x_3); lean_ctor_set(x_5, 1, x_4); x_6 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_7 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_5, x_6); +x_7 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_5, x_6); x_8 = l_Lean_Json_mkObj(x_7); return x_8; } @@ -22473,7 +22473,7 @@ x_5 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_5, 0, x_3); lean_ctor_set(x_5, 1, x_4); x_6 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_7 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_5, x_6); +x_7 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_5, x_6); x_8 = l_Lean_Json_mkObj(x_7); return x_8; } @@ -23147,7 +23147,7 @@ x_11 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_11, 0, x_10); lean_ctor_set(x_11, 1, x_9); x_12 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_13 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_11, x_12); +x_13 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_11, x_12); x_14 = l_Lean_Json_mkObj(x_13); return x_14; } @@ -23159,7 +23159,7 @@ x_16 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_16, 0, x_15); lean_ctor_set(x_16, 1, x_9); x_17 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_18 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_16, x_17); +x_18 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_16, x_17); x_19 = l_Lean_Json_mkObj(x_18); return x_19; } @@ -23515,7 +23515,7 @@ x_15 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_15, 0, x_9); lean_ctor_set(x_15, 1, x_14); x_16 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_17 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_15, x_16); +x_17 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_15, x_16); x_18 = l_Lean_Json_mkObj(x_17); return x_18; } @@ -23552,7 +23552,7 @@ x_31 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_31, 0, x_25); lean_ctor_set(x_31, 1, x_30); x_32 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_33 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_31, x_32); +x_33 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_31, x_32); x_34 = l_Lean_Json_mkObj(x_33); return x_34; } @@ -23655,7 +23655,7 @@ x_22 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_22, 0, x_10); lean_ctor_set(x_22, 1, x_21); x_23 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_24 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_22, x_23); +x_24 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_22, x_23); x_25 = l_Lean_Json_mkObj(x_24); return x_25; } @@ -23741,7 +23741,7 @@ x_29 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_29, 0, x_11); lean_ctor_set(x_29, 1, x_28); x_30 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_31 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_29, x_30); +x_31 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_29, x_30); x_32 = l_Lean_Json_mkObj(x_31); return x_32; } @@ -23790,7 +23790,7 @@ x_12 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_12, 0, x_8); lean_ctor_set(x_12, 1, x_11); x_13 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_14 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); +x_14 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); x_15 = l_Lean_Json_mkObj(x_14); return x_15; } @@ -23821,7 +23821,7 @@ x_26 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_26, 0, x_22); lean_ctor_set(x_26, 1, x_25); x_27 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_28 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_26, x_27); +x_28 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_26, x_27); x_29 = l_Lean_Json_mkObj(x_28); return x_29; } @@ -23909,7 +23909,7 @@ x_5 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_5, 0, x_3); lean_ctor_set(x_5, 1, x_4); x_6 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_7 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_5, x_6); +x_7 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_5, x_6); x_8 = l_Lean_Json_mkObj(x_7); return x_8; } @@ -24288,7 +24288,7 @@ x_5 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_5, 0, x_3); lean_ctor_set(x_5, 1, x_4); x_6 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_7 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_5, x_6); +x_7 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_5, x_6); x_8 = l_Lean_Json_mkObj(x_7); return x_8; } @@ -24495,7 +24495,7 @@ x_7 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_7, 0, x_6); lean_ctor_set(x_7, 1, x_5); x_8 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } diff --git a/stage0/stdlib/Lean/Data/Lsp/Capabilities.c b/stage0/stdlib/Lean/Data/Lsp/Capabilities.c index ee189634c2c9..9cdb88c2fba3 100644 --- a/stage0/stdlib/Lean/Data/Lsp/Capabilities.c +++ b/stage0/stdlib/Lean/Data/Lsp/Capabilities.c @@ -92,6 +92,7 @@ static lean_object* l_Lean_Lsp_instFromJsonWindowClientCapabilities___closed__1; lean_object* l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_fromJsonCodeActionOptions____x40_Lean_Data_Lsp_CodeActions___hyg_884_(lean_object*); static lean_object* l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_toJsonWorkspaceClientCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_963____closed__1; LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_toJsonServerCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_1460____spec__2(lean_object*, lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_fromJsonWorkspaceEditClientCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_794____closed__7; static lean_object* l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_fromJsonCompletionItemCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_48____closed__2; static lean_object* l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_fromJsonChangeAnnotationSupport____x40_Lean_Data_Lsp_Capabilities___hyg_654____closed__6; @@ -216,7 +217,6 @@ LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_Capabiliti static lean_object* l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_fromJsonServerCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_1644____closed__53; static lean_object* l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_fromJsonServerCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_1644____closed__33; LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonCompletionItemCapabilities; -lean_object* l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_toJsonTextDocumentClientCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_248____spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_toJsonWorkspaceClientCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_963_(lean_object*); static lean_object* l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_fromJsonCompletionItemCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_48____closed__13; @@ -393,7 +393,7 @@ x_5 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_5, 0, x_3); lean_ctor_set(x_5, 1, x_4); x_6 = l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_toJsonCompletionItemCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_20____closed__2; -x_7 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_5, x_6); +x_7 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_5, x_6); x_8 = l_Lean_Json_mkObj(x_7); return x_8; } @@ -686,7 +686,7 @@ x_5 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_5, 0, x_3); lean_ctor_set(x_5, 1, x_4); x_6 = l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_toJsonCompletionItemCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_20____closed__2; -x_7 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_5, x_6); +x_7 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_5, x_6); x_8 = l_Lean_Json_mkObj(x_7); return x_8; } @@ -1166,7 +1166,7 @@ x_10 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_10, 0, x_4); lean_ctor_set(x_10, 1, x_9); x_11 = l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_toJsonCompletionItemCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_20____closed__2; -x_12 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_10, x_11); +x_12 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_10, x_11); x_13 = l_Lean_Json_mkObj(x_12); return x_13; } @@ -1838,7 +1838,7 @@ x_7 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_7, 0, x_6); lean_ctor_set(x_7, 1, x_5); x_8 = l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_toJsonCompletionItemCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_20____closed__2; -x_9 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -2070,7 +2070,7 @@ x_5 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_5, 0, x_3); lean_ctor_set(x_5, 1, x_4); x_6 = l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_toJsonCompletionItemCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_20____closed__2; -x_7 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_5, x_6); +x_7 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_5, x_6); x_8 = l_Lean_Json_mkObj(x_7); return x_8; } @@ -2449,7 +2449,7 @@ x_5 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_5, 0, x_3); lean_ctor_set(x_5, 1, x_4); x_6 = l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_toJsonCompletionItemCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_20____closed__2; -x_7 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_5, x_6); +x_7 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_5, x_6); x_8 = l_Lean_Json_mkObj(x_7); return x_8; } @@ -2719,7 +2719,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_4); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_toJsonCompletionItemCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_20____closed__2; -x_16 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -3344,7 +3344,7 @@ x_10 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_10, 0, x_4); lean_ctor_set(x_10, 1, x_9); x_11 = l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_toJsonCompletionItemCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_20____closed__2; -x_12 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_10, x_11); +x_12 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_10, x_11); x_13 = l_Lean_Json_mkObj(x_12); return x_13; } @@ -3938,7 +3938,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_4); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_toJsonCompletionItemCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_20____closed__2; -x_16 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -5280,7 +5280,7 @@ x_82 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_82, 0, x_4); lean_ctor_set(x_82, 1, x_81); x_83 = l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_toJsonCompletionItemCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_20____closed__2; -x_84 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_82, x_83); +x_84 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_82, x_83); x_85 = l_Lean_Json_mkObj(x_84); return x_85; } diff --git a/stage0/stdlib/Lean/Data/Lsp/Client.c b/stage0/stdlib/Lean/Data/Lsp/Client.c index 2759c97dee51..51a4f39710a6 100644 --- a/stage0/stdlib/Lean/Data/Lsp/Client.c +++ b/stage0/stdlib/Lean/Data/Lsp/Client.c @@ -44,6 +44,7 @@ static lean_object* l___private_Lean_Data_Lsp_Client_0__Lean_Lsp_fromJsonRegistr static lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Client_0__Lean_Lsp_fromJsonRegistrationParams____x40_Lean_Data_Lsp_Client___hyg_296____spec__1___closed__1; lean_object* l_Lean_Json_getObjValD(lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Data_Lsp_Client_0__Lean_Lsp_fromJsonRegistration____x40_Lean_Data_Lsp_Client___hyg_100____lambda__1(lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_Client_0__Lean_Lsp_toJsonRegistration____x40_Lean_Data_Lsp_Client___hyg_34____closed__5; static lean_object* l___private_Lean_Data_Lsp_Client_0__Lean_Lsp_fromJsonRegistrationParams____x40_Lean_Data_Lsp_Client___hyg_296____closed__2; LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonRegistration; @@ -52,7 +53,6 @@ static lean_object* l___private_Lean_Data_Lsp_Client_0__Lean_Lsp_fromJsonRegistr LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_Client_0__Lean_Lsp_fromJsonRegistration____x40_Lean_Data_Lsp_Client___hyg_100_(lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_Client_0__Lean_Lsp_toJsonRegistrationParams____x40_Lean_Data_Lsp_Client___hyg_258____closed__1; -lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_Client_0__Lean_Lsp_fromJsonRegistration____x40_Lean_Data_Lsp_Client___hyg_100____closed__2; static lean_object* l___private_Lean_Data_Lsp_Client_0__Lean_Lsp_fromJsonRegistration____x40_Lean_Data_Lsp_Client___hyg_100____closed__10; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_Client_0__Lean_Lsp_fromJsonRegistrationParams____x40_Lean_Data_Lsp_Client___hyg_296____spec__2(size_t, size_t, lean_object*); @@ -199,7 +199,7 @@ x_16 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_16, 0, x_9); lean_ctor_set(x_16, 1, x_15); x_17 = l___private_Lean_Data_Lsp_Client_0__Lean_Lsp_toJsonRegistration____x40_Lean_Data_Lsp_Client___hyg_34____closed__3; -x_18 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_16, x_17); +x_18 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_16, x_17); x_19 = l_Lean_Json_mkObj(x_18); return x_19; } @@ -225,7 +225,7 @@ x_26 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_26, 0, x_9); lean_ctor_set(x_26, 1, x_25); x_27 = l___private_Lean_Data_Lsp_Client_0__Lean_Lsp_toJsonRegistration____x40_Lean_Data_Lsp_Client___hyg_34____closed__3; -x_28 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_26, x_27); +x_28 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_26, x_27); x_29 = l_Lean_Json_mkObj(x_28); return x_29; } @@ -702,7 +702,7 @@ x_10 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_10, 0, x_9); lean_ctor_set(x_10, 1, x_8); x_11 = l___private_Lean_Data_Lsp_Client_0__Lean_Lsp_toJsonRegistration____x40_Lean_Data_Lsp_Client___hyg_34____closed__3; -x_12 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_10, x_11); +x_12 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_10, x_11); x_13 = l_Lean_Json_mkObj(x_12); return x_13; } diff --git a/stage0/stdlib/Lean/Data/Lsp/CodeActions.c b/stage0/stdlib/Lean/Data/Lsp/CodeActions.c index 5f4143d78cec..0d646703d94f 100644 --- a/stage0/stdlib/Lean/Data/Lsp/CodeActions.c +++ b/stage0/stdlib/Lean/Data/Lsp/CodeActions.c @@ -96,6 +96,7 @@ LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Ls static lean_object* l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_fromJsonCodeActionLiteralSupportValueSet____x40_Lean_Data_Lsp_CodeActions___hyg_1753____closed__3; static lean_object* l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_fromJsonCodeActionClientCapabilities____x40_Lean_Data_Lsp_CodeActions___hyg_2049____closed__43; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_fromJsonCodeAction____x40_Lean_Data_Lsp_CodeActions___hyg_1204_(lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_fromJsonCodeActionDisabled____x40_Lean_Data_Lsp_CodeActions___hyg_698____closed__7; static lean_object* l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_fromJsonCodeActionClientCapabilities____x40_Lean_Data_Lsp_CodeActions___hyg_2049____closed__9; static lean_object* l_Lean_Lsp_CodeActionTriggerKind_noConfusion___rarg___closed__1; @@ -262,7 +263,6 @@ static lean_object* l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_fromJsonCo static lean_object* l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_fromJsonCodeActionClientCapabilities____x40_Lean_Data_Lsp_CodeActions___hyg_2049____closed__22; static lean_object* l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_fromJsonCodeActionClientCapabilities____x40_Lean_Data_Lsp_CodeActions___hyg_2049____closed__12; static lean_object* l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_fromJsonCodeActionLiteralSupportValueSet____x40_Lean_Data_Lsp_CodeActions___hyg_1753____closed__8; -lean_object* l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_fromJsonCodeActionOptions____x40_Lean_Data_Lsp_CodeActions___hyg_884____closed__15; static lean_object* l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_fromJsonCodeAction____x40_Lean_Data_Lsp_CodeActions___hyg_1204____closed__12; LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonCodeActionContext; @@ -1742,7 +1742,7 @@ x_19 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_19, 0, x_10); lean_ctor_set(x_19, 1, x_18); x_20 = l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_toJsonCodeActionContext____x40_Lean_Data_Lsp_CodeActions___hyg_292____closed__1; -x_21 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_19, x_20); +x_21 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_19, x_20); x_22 = l_Lean_Json_mkObj(x_21); return x_22; } @@ -2415,7 +2415,7 @@ x_28 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_28, 0, x_4); lean_ctor_set(x_28, 1, x_27); x_29 = l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_toJsonCodeActionContext____x40_Lean_Data_Lsp_CodeActions___hyg_292____closed__1; -x_30 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_28, x_29); +x_30 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_28, x_29); x_31 = l_Lean_Json_mkObj(x_30); return x_31; } @@ -2614,7 +2614,7 @@ x_7 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_7, 0, x_6); lean_ctor_set(x_7, 1, x_5); x_8 = l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_toJsonCodeActionContext____x40_Lean_Data_Lsp_CodeActions___hyg_292____closed__1; -x_9 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -2725,7 +2725,7 @@ x_17 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_17, 0, x_10); lean_ctor_set(x_17, 1, x_16); x_18 = l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_toJsonCodeActionContext____x40_Lean_Data_Lsp_CodeActions___hyg_292____closed__1; -x_19 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_17, x_18); +x_19 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_17, x_18); x_20 = l_Lean_Json_mkObj(x_19); return x_20; } @@ -3604,7 +3604,7 @@ x_44 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_44, 0, x_4); lean_ctor_set(x_44, 1, x_43); x_45 = l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_toJsonCodeActionContext____x40_Lean_Data_Lsp_CodeActions___hyg_292____closed__1; -x_46 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_44, x_45); +x_46 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_44, x_45); x_47 = l_Lean_Json_mkObj(x_46); return x_47; } @@ -5806,7 +5806,7 @@ x_10 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_10, 0, x_9); lean_ctor_set(x_10, 1, x_8); x_11 = l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_toJsonCodeActionContext____x40_Lean_Data_Lsp_CodeActions___hyg_292____closed__1; -x_12 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_10, x_11); +x_12 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_10, x_11); x_13 = l_Lean_Json_mkObj(x_12); return x_13; } @@ -6112,7 +6112,7 @@ x_10 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_10, 0, x_9); lean_ctor_set(x_10, 1, x_8); x_11 = l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_toJsonCodeActionContext____x40_Lean_Data_Lsp_CodeActions___hyg_292____closed__1; -x_12 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_10, x_11); +x_12 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_10, x_11); x_13 = l_Lean_Json_mkObj(x_12); return x_13; } @@ -6328,7 +6328,7 @@ x_7 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_7, 0, x_6); lean_ctor_set(x_7, 1, x_5); x_8 = l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_toJsonCodeActionContext____x40_Lean_Data_Lsp_CodeActions___hyg_292____closed__1; -x_9 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -7608,7 +7608,7 @@ x_30 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_30, 0, x_4); lean_ctor_set(x_30, 1, x_29); x_31 = l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_toJsonCodeActionContext____x40_Lean_Data_Lsp_CodeActions___hyg_292____closed__1; -x_32 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_30, x_31); +x_32 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_30, x_31); x_33 = l_Lean_Json_mkObj(x_32); return x_33; } diff --git a/stage0/stdlib/Lean/Data/Lsp/Diagnostics.c b/stage0/stdlib/Lean/Data/Lsp/Diagnostics.c index 4556dc51d242..f0faf487387c 100644 --- a/stage0/stdlib/Lean/Data/Lsp/Diagnostics.c +++ b/stage0/stdlib/Lean/Data/Lsp/Diagnostics.c @@ -90,6 +90,7 @@ lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Basic_0__L static lean_object* l_Lean_Lsp_instToJsonDiagnosticSeverity___closed__5; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_beqDiagnosticTag____x40_Lean_Data_Lsp_Diagnostics___hyg_625____boxed(lean_object*, lean_object*); static lean_object* l_Lean_Lsp_instFromJsonDiagnosticCode___closed__1; +lean_object* l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_DiagnosticWith_ordUserVisible____x40_Lean_Data_Lsp_Diagnostics___hyg_2053____rarg___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_fromJsonDiagnosticWith____x40_Lean_Data_Lsp_Diagnostics___hyg_1550____rarg___closed__25; static lean_object* l___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_fromJsonDiagnosticWith____x40_Lean_Data_Lsp_Diagnostics___hyg_1550____rarg___closed__19; @@ -219,7 +220,6 @@ static lean_object* l_Lean_Lsp_instFromJsonDiagnosticSeverity___closed__3; static lean_object* l___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_fromJsonDiagnosticWith____x40_Lean_Data_Lsp_Diagnostics___hyg_1550____rarg___closed__40; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_DiagnosticWith_UserVisible_ofDiagnostic___rarg(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_toJsonDiagnosticWith____x40_Lean_Data_Lsp_Diagnostics___hyg_1452_(lean_object*); -lean_object* l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_ordDiagnosticCode____x40_Lean_Data_Lsp_Diagnostics___hyg_404____boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_compareByUserVisible(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_toJsonPublishDiagnosticsParams____x40_Lean_Data_Lsp_Diagnostics___hyg_2411____spec__3(size_t, size_t, lean_object*); @@ -1905,7 +1905,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_7); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_toJsonDiagnosticRelatedInformation____x40_Lean_Data_Lsp_Diagnostics___hyg_901____closed__3; -x_16 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -3548,7 +3548,7 @@ x_43 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_43, 0, x_8); lean_ctor_set(x_43, 1, x_42); x_44 = l___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_toJsonDiagnosticRelatedInformation____x40_Lean_Data_Lsp_Diagnostics___hyg_901____closed__3; -x_45 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_43, x_44); +x_45 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_43, x_44); x_46 = l_Lean_Json_mkObj(x_45); return x_46; } @@ -6883,7 +6883,7 @@ x_42 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_42, 0, x_7); lean_ctor_set(x_42, 1, x_41); x_43 = l___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_toJsonDiagnosticRelatedInformation____x40_Lean_Data_Lsp_Diagnostics___hyg_901____closed__3; -x_44 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_42, x_43); +x_44 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_42, x_43); x_45 = l_Lean_Json_mkObj(x_44); return x_45; } @@ -6982,7 +6982,7 @@ x_21 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_21, 0, x_9); lean_ctor_set(x_21, 1, x_20); x_22 = l___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_toJsonDiagnosticRelatedInformation____x40_Lean_Data_Lsp_Diagnostics___hyg_901____closed__3; -x_23 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_21, x_22); +x_23 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_21, x_22); x_24 = l_Lean_Json_mkObj(x_23); return x_24; } diff --git a/stage0/stdlib/Lean/Data/Lsp/Extra.c b/stage0/stdlib/Lean/Data/Lsp/Extra.c index 30f8532feeaf..c5828e88b977 100644 --- a/stage0/stdlib/Lean/Data/Lsp/Extra.c +++ b/stage0/stdlib/Lean/Data/Lsp/Extra.c @@ -110,6 +110,7 @@ static lean_object* l_Lean_Lsp_instToJsonPlainTermGoalParams___closed__1; static lean_object* l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonRpcCallParams____x40_Lean_Data_Lsp_Extra___hyg_2012____closed__6; static lean_object* l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonPlainTermGoal____x40_Lean_Data_Lsp_Extra___hyg_1584____closed__4; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_toJsonLeanFileProgressProcessingInfo____x40_Lean_Data_Lsp_Extra___hyg_814_(lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonRpcConnected____x40_Lean_Data_Lsp_Extra___hyg_1871____spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Lsp_instReprLineRange___closed__1; lean_object* l___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173_(size_t); @@ -272,7 +273,6 @@ static lean_object* l_Lean_Lsp_instFromJsonRpcKeepAliveParams___closed__1; static lean_object* l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_toJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_132____closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_toJsonPlainGoal____x40_Lean_Data_Lsp_Extra___hyg_1342____spec__1(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonRpcReleaseParams; -lean_object* l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonRpcCallParams____x40_Lean_Data_Lsp_Extra___hyg_2012____closed__15; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____lambda__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonDependencyBuildMode; @@ -1496,7 +1496,7 @@ x_12 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_12, 0, x_7); lean_ctor_set(x_12, 1, x_11); x_13 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_14 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_12, x_13); +x_14 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_12, x_13); x_15 = l_Lean_Json_mkObj(x_14); return x_15; } @@ -1811,7 +1811,7 @@ x_15 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_15, 0, x_8); lean_ctor_set(x_15, 1, x_14); x_16 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_17 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_15, x_16); +x_17 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_15, x_16); x_18 = l_Lean_Json_mkObj(x_17); return x_18; } @@ -1850,7 +1850,7 @@ x_32 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_32, 0, x_25); lean_ctor_set(x_32, 1, x_31); x_33 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_34 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_32, x_33); +x_34 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_32, x_33); x_35 = l_Lean_Json_mkObj(x_34); return x_35; } @@ -2828,7 +2828,7 @@ x_10 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_10, 0, x_7); lean_ctor_set(x_10, 1, x_9); x_11 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_12 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_10, x_11); +x_12 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_10, x_11); x_13 = l_Lean_Json_mkObj(x_12); return x_13; } @@ -2840,7 +2840,7 @@ x_15 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_15, 0, x_7); lean_ctor_set(x_15, 1, x_14); x_16 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_17 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_15, x_16); +x_17 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_15, x_16); x_18 = l_Lean_Json_mkObj(x_17); return x_18; } @@ -3320,7 +3320,7 @@ x_17 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_17, 0, x_7); lean_ctor_set(x_17, 1, x_16); x_18 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_19 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_17, x_18); +x_19 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_17, x_18); x_20 = l_Lean_Json_mkObj(x_19); return x_20; } @@ -3615,7 +3615,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_7); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -4117,7 +4117,7 @@ x_17 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_17, 0, x_8); lean_ctor_set(x_17, 1, x_16); x_18 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_19 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_17, x_18); +x_19 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_17, x_18); x_20 = l_Lean_Json_mkObj(x_19); return x_20; } @@ -4158,7 +4158,7 @@ x_36 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_36, 0, x_27); lean_ctor_set(x_36, 1, x_35); x_37 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_38 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_36, x_37); +x_38 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_36, x_37); x_39 = l_Lean_Json_mkObj(x_38); return x_39; } @@ -4425,7 +4425,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_7); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -4709,7 +4709,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_8); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -4746,7 +4746,7 @@ x_30 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_30, 0, x_24); lean_ctor_set(x_30, 1, x_29); x_31 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_32 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_30, x_31); +x_32 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_30, x_31); x_33 = l_Lean_Json_mkObj(x_32); return x_33; } @@ -4917,7 +4917,7 @@ x_7 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_7, 0, x_6); lean_ctor_set(x_7, 1, x_5); x_8 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_9 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -5223,7 +5223,7 @@ x_8 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_8, 0, x_7); lean_ctor_set(x_8, 1, x_6); x_9 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_10 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_8, x_9); +x_10 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_8, x_9); x_11 = l_Lean_Json_mkObj(x_10); return x_11; } @@ -5949,7 +5949,7 @@ x_36 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_36, 0, x_8); lean_ctor_set(x_36, 1, x_35); x_37 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_38 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_36, x_37); +x_38 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_36, x_37); x_39 = l_Lean_Json_mkObj(x_38); return x_39; } @@ -6503,7 +6503,7 @@ x_24 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_24, 0, x_9); lean_ctor_set(x_24, 1, x_23); x_25 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_26 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_24, x_25); +x_26 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_24, x_25); x_27 = l_Lean_Json_mkObj(x_26); return x_27; } @@ -6773,7 +6773,7 @@ x_15 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_15, 0, x_8); lean_ctor_set(x_15, 1, x_14); x_16 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_17 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_15, x_16); +x_17 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_15, x_16); x_18 = l_Lean_Json_mkObj(x_17); return x_18; } @@ -7365,7 +7365,7 @@ x_16 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_16, 0, x_8); lean_ctor_set(x_16, 1, x_15); x_17 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_18 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_16, x_17); +x_18 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_16, x_17); x_19 = l_Lean_Json_mkObj(x_18); return x_19; } diff --git a/stage0/stdlib/Lean/Data/Lsp/InitShutdown.c b/stage0/stdlib/Lean/Data/Lsp/InitShutdown.c index f86a5fe5ceb7..267e8d587b9b 100644 --- a/stage0/stdlib/Lean/Data/Lsp/InitShutdown.c +++ b/stage0/stdlib/Lean/Data/Lsp/InitShutdown.c @@ -61,6 +61,7 @@ static lean_object* l___private_Lean_Data_Lsp_InitShutdown_0__Lean_Lsp_fromJsonI LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_InitShutdown_0__Lean_Lsp_fromJsonInitializeResult____x40_Lean_Data_Lsp_InitShutdown___hyg_966____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_InitShutdown_0__Lean_Lsp_toJsonInitializeParams____x40_Lean_Data_Lsp_InitShutdown___hyg_522____closed__2; static lean_object* l_Lean_Lsp_Trace_noConfusion___rarg___closed__1; +lean_object* l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); uint8_t lean_string_dec_eq(lean_object*, lean_object*); static lean_object* l_Lean_Json_getObjValAs_x3f___at_Lean_Lsp_instFromJsonInitializeParams___spec__6___closed__1; lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonVersionedTextDocumentIdentifier____x40_Lean_Data_Lsp_Basic___hyg_2438____spec__1(lean_object*, lean_object*); @@ -129,7 +130,6 @@ lean_object* l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_fromJsonClientCa LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at_Lean_Lsp_instFromJsonInitializeParams___spec__5___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at_Lean_Lsp_instFromJsonInitializeParams___spec__3___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_InitShutdown_0__Lean_Lsp_fromJsonInitializationOptions____x40_Lean_Data_Lsp_InitShutdown___hyg_342____closed__10; -lean_object* l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_InitShutdown_0__Lean_Lsp_toJsonClientInfo____x40_Lean_Data_Lsp_InitShutdown___hyg_28____closed__3; static lean_object* l___private_Lean_Data_Lsp_InitShutdown_0__Lean_Lsp_fromJsonServerInfo____x40_Lean_Data_Lsp_InitShutdown___hyg_796____closed__4; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_InitShutdown_0__Lean_Lsp_fromJsonClientInfo____x40_Lean_Data_Lsp_InitShutdown___hyg_70____lambda__1___boxed(lean_object*); @@ -261,7 +261,7 @@ x_12 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_12, 0, x_8); lean_ctor_set(x_12, 1, x_11); x_13 = l___private_Lean_Data_Lsp_InitShutdown_0__Lean_Lsp_toJsonClientInfo____x40_Lean_Data_Lsp_InitShutdown___hyg_28____closed__3; -x_14 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_12, x_13); +x_14 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_12, x_13); x_15 = l_Lean_Json_mkObj(x_14); return x_15; } @@ -292,7 +292,7 @@ x_26 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_26, 0, x_22); lean_ctor_set(x_26, 1, x_25); x_27 = l___private_Lean_Data_Lsp_InitShutdown_0__Lean_Lsp_toJsonClientInfo____x40_Lean_Data_Lsp_InitShutdown___hyg_28____closed__3; -x_28 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_26, x_27); +x_28 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_26, x_27); x_29 = l_Lean_Json_mkObj(x_28); return x_29; } @@ -949,7 +949,7 @@ x_10 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_10, 0, x_4); lean_ctor_set(x_10, 1, x_9); x_11 = l___private_Lean_Data_Lsp_InitShutdown_0__Lean_Lsp_toJsonClientInfo____x40_Lean_Data_Lsp_InitShutdown___hyg_28____closed__3; -x_12 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_10, x_11); +x_12 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_10, x_11); x_13 = l_Lean_Json_mkObj(x_12); return x_13; } @@ -1556,7 +1556,7 @@ x_31 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_31, 0, x_4); lean_ctor_set(x_31, 1, x_30); x_32 = l___private_Lean_Data_Lsp_InitShutdown_0__Lean_Lsp_toJsonClientInfo____x40_Lean_Data_Lsp_InitShutdown___hyg_28____closed__3; -x_33 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_31, x_32); +x_33 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_31, x_32); x_34 = l_Lean_Json_mkObj(x_33); return x_34; } @@ -1583,7 +1583,7 @@ x_41 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_41, 0, x_4); lean_ctor_set(x_41, 1, x_40); x_42 = l___private_Lean_Data_Lsp_InitShutdown_0__Lean_Lsp_toJsonClientInfo____x40_Lean_Data_Lsp_InitShutdown___hyg_28____closed__3; -x_43 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_41, x_42); +x_43 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_41, x_42); x_44 = l_Lean_Json_mkObj(x_43); return x_44; } @@ -1610,7 +1610,7 @@ x_51 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_51, 0, x_4); lean_ctor_set(x_51, 1, x_50); x_52 = l___private_Lean_Data_Lsp_InitShutdown_0__Lean_Lsp_toJsonClientInfo____x40_Lean_Data_Lsp_InitShutdown___hyg_28____closed__3; -x_53 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_51, x_52); +x_53 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_51, x_52); x_54 = l_Lean_Json_mkObj(x_53); return x_54; } @@ -4199,7 +4199,7 @@ x_12 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_12, 0, x_8); lean_ctor_set(x_12, 1, x_11); x_13 = l___private_Lean_Data_Lsp_InitShutdown_0__Lean_Lsp_toJsonClientInfo____x40_Lean_Data_Lsp_InitShutdown___hyg_28____closed__3; -x_14 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_12, x_13); +x_14 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_12, x_13); x_15 = l_Lean_Json_mkObj(x_14); return x_15; } @@ -4230,7 +4230,7 @@ x_26 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_26, 0, x_22); lean_ctor_set(x_26, 1, x_25); x_27 = l___private_Lean_Data_Lsp_InitShutdown_0__Lean_Lsp_toJsonClientInfo____x40_Lean_Data_Lsp_InitShutdown___hyg_28____closed__3; -x_28 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_26, x_27); +x_28 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_26, x_27); x_29 = l_Lean_Json_mkObj(x_28); return x_29; } @@ -4515,7 +4515,7 @@ x_12 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_12, 0, x_7); lean_ctor_set(x_12, 1, x_11); x_13 = l___private_Lean_Data_Lsp_InitShutdown_0__Lean_Lsp_toJsonClientInfo____x40_Lean_Data_Lsp_InitShutdown___hyg_28____closed__3; -x_14 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_12, x_13); +x_14 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_12, x_13); x_15 = l_Lean_Json_mkObj(x_14); return x_15; } diff --git a/stage0/stdlib/Lean/Data/Lsp/Internal.c b/stage0/stdlib/Lean/Data/Lsp/Internal.c index 5f2a5fcb6091..df2d810cb271 100644 --- a/stage0/stdlib/Lean/Data/Lsp/Internal.c +++ b/stage0/stdlib/Lean/Data/Lsp/Internal.c @@ -117,6 +117,7 @@ LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonRefInfo(lean_object*); static lean_object* l_Lean_Lsp_instInhabitedRefIdent___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instToJsonModuleRefs___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_RBNode_foldM___at_Lean_Lsp_instFromJsonModuleRefs___spec__6___closed__1; +lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_toJsonLeanIleanInfoParams____x40_Lean_Data_Lsp_Internal___hyg_1979____spec__2(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_RefIdent_fromJsonRefIdentJsonRepr____x40_Lean_Data_Lsp_Internal___hyg_268____lambda__1___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Lsp_instToJsonModuleRefs___spec__4(lean_object*, size_t, size_t, lean_object*); @@ -135,7 +136,6 @@ static lean_object* l_Lean_Lsp_instToJsonRefInfo___closed__3; static lean_object* l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_fromJsonLeanStaleDependencyParams____x40_Lean_Data_Lsp_Internal___hyg_2161____closed__4; LEAN_EXPORT lean_object* l_Lean_Lsp_RefIdent_fromJson_x3f(lean_object*); static lean_object* l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_fromJsonLeanIleanInfoParams____x40_Lean_Data_Lsp_Internal___hyg_1873____closed__8; -lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_fromJsonLeanIleanInfoParams____x40_Lean_Data_Lsp_Internal___hyg_1873____closed__13; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instFromJsonRefInfo___spec__2___closed__1; static lean_object* l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_fromJsonLeanIleanInfoParams____x40_Lean_Data_Lsp_Internal___hyg_1873____closed__19; @@ -1805,7 +1805,7 @@ x_20 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_20, 0, x_9); lean_ctor_set(x_20, 1, x_19); x_21 = l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_RefInfo_toJsonParentDecl____x40_Lean_Data_Lsp_Internal___hyg_721____closed__4; -x_22 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_20, x_21); +x_22 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_20, x_21); x_23 = l_Lean_Json_mkObj(x_22); return x_23; } @@ -16575,7 +16575,7 @@ x_20 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_20, 0, x_8); lean_ctor_set(x_20, 1, x_19); x_21 = l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_RefInfo_toJsonParentDecl____x40_Lean_Data_Lsp_Internal___hyg_721____closed__4; -x_22 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_20, x_21); +x_22 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_20, x_21); x_23 = l_Lean_Json_mkObj(x_22); return x_23; } @@ -16604,7 +16604,7 @@ x_31 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_31, 0, x_8); lean_ctor_set(x_31, 1, x_30); x_32 = l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_RefInfo_toJsonParentDecl____x40_Lean_Data_Lsp_Internal___hyg_721____closed__4; -x_33 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_31, x_32); +x_33 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_31, x_32); x_34 = l_Lean_Json_mkObj(x_33); return x_34; } @@ -16632,7 +16632,7 @@ x_44 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_44, 0, x_8); lean_ctor_set(x_44, 1, x_43); x_45 = l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_RefInfo_toJsonParentDecl____x40_Lean_Data_Lsp_Internal___hyg_721____closed__4; -x_46 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_44, x_45); +x_46 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_44, x_45); x_47 = l_Lean_Json_mkObj(x_46); return x_47; } @@ -17035,7 +17035,7 @@ x_10 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_10, 0, x_9); lean_ctor_set(x_10, 1, x_8); x_11 = l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_RefInfo_toJsonParentDecl____x40_Lean_Data_Lsp_Internal___hyg_721____closed__4; -x_12 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_10, x_11); +x_12 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_10, x_11); x_13 = l_Lean_Json_mkObj(x_12); return x_13; } @@ -17246,7 +17246,7 @@ x_7 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_7, 0, x_6); lean_ctor_set(x_7, 1, x_5); x_8 = l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_RefInfo_toJsonParentDecl____x40_Lean_Data_Lsp_Internal___hyg_721____closed__4; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } diff --git a/stage0/stdlib/Lean/Data/Lsp/LanguageFeatures.c b/stage0/stdlib/Lean/Data/Lsp/LanguageFeatures.c index 38505f3c21f4..40b423c9bb62 100644 --- a/stage0/stdlib/Lean/Data/Lsp/LanguageFeatures.c +++ b/stage0/stdlib/Lean/Data/Lsp/LanguageFeatures.c @@ -675,6 +675,7 @@ static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJ static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1756____closed__5; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1756____closed__49; static lean_object* l_Lean_Lsp_SemanticTokenType_names___closed__8; +lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonDocumentHighlightParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3855____closed__6; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_7320____closed__10; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonHoverParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2816_(lean_object*); @@ -789,7 +790,6 @@ static lean_object* l_Lean_Lsp_instToJsonDocumentHighlightKind___closed__3; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonRenameParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_10390____closed__9; LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonDocumentSymbol_go(lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_348____closed__110; -lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonDocumentSymbolAux(lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_9149____closed__2; @@ -2272,7 +2272,7 @@ x_16 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_16, 0, x_4); lean_ctor_set(x_16, 1, x_15); x_17 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_18 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_16, x_17); +x_18 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_16, x_17); x_19 = l_Lean_Json_mkObj(x_18); return x_19; } @@ -5537,7 +5537,7 @@ x_20 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_20, 0, x_9); lean_ctor_set(x_20, 1, x_19); x_21 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_22 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_20, x_21); +x_22 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_20, x_21); x_23 = l_Lean_Json_mkObj(x_22); return x_23; } @@ -7820,7 +7820,7 @@ x_36 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_36, 0, x_14); lean_ctor_set(x_36, 1, x_35); x_37 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_38 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_36, x_37); +x_38 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_36, x_37); x_39 = l_Lean_Json_mkObj(x_38); return x_39; } @@ -8379,7 +8379,7 @@ x_17 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_17, 0, x_8); lean_ctor_set(x_17, 1, x_16); x_18 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_19 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_17, x_18); +x_19 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_17, x_18); x_20 = l_Lean_Json_mkObj(x_19); return x_20; } @@ -8703,7 +8703,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_7); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -8768,7 +8768,7 @@ x_12 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_12, 0, x_7); lean_ctor_set(x_12, 1, x_11); x_13 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_14 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); +x_14 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); x_15 = l_Lean_Json_mkObj(x_14); return x_15; } @@ -9290,7 +9290,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_7); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -9544,7 +9544,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_7); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -9798,7 +9798,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_7); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -10052,7 +10052,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_7); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -10251,7 +10251,7 @@ x_7 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_7, 0, x_6); lean_ctor_set(x_7, 1, x_5); x_8 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -10647,7 +10647,7 @@ x_22 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_22, 0, x_8); lean_ctor_set(x_22, 1, x_21); x_23 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_24 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_22, x_23); +x_24 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_22, x_23); x_25 = l_Lean_Json_mkObj(x_24); return x_25; } @@ -10846,7 +10846,7 @@ x_7 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_7, 0, x_6); lean_ctor_set(x_7, 1, x_5); x_8 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -11100,7 +11100,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_7); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -11342,7 +11342,7 @@ x_12 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_12, 0, x_7); lean_ctor_set(x_12, 1, x_11); x_13 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_14 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); +x_14 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); x_15 = l_Lean_Json_mkObj(x_14); return x_15; } @@ -11520,7 +11520,7 @@ x_7 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_7, 0, x_6); lean_ctor_set(x_7, 1, x_5); x_8 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -21351,7 +21351,7 @@ x_35 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_35, 0, x_13); lean_ctor_set(x_35, 1, x_34); x_36 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_37 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_35, x_36); +x_37 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_35, x_36); x_38 = l_Lean_Json_mkObj(x_37); return x_38; } @@ -21733,7 +21733,7 @@ x_34 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_34, 0, x_12); lean_ctor_set(x_34, 1, x_33); x_35 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_36 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_34, x_35); +x_36 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_34, x_35); x_37 = l_Lean_Json_mkObj(x_36); return x_37; } @@ -23360,7 +23360,7 @@ x_33 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_33, 0, x_11); lean_ctor_set(x_33, 1, x_32); x_34 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_35 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_33, x_34); +x_35 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_33, x_34); x_36 = l_Lean_Json_mkObj(x_35); return x_36; } @@ -23627,7 +23627,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_7); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -24755,7 +24755,7 @@ x_44 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_44, 0, x_14); lean_ctor_set(x_44, 1, x_43); x_45 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_46 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_44, x_45); +x_46 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_44, x_45); x_47 = l_Lean_Json_mkObj(x_46); return x_47; } @@ -25552,7 +25552,7 @@ x_7 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_7, 0, x_6); lean_ctor_set(x_7, 1, x_5); x_8 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -26052,7 +26052,7 @@ x_17 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_17, 0, x_7); lean_ctor_set(x_17, 1, x_16); x_18 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_19 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_17, x_18); +x_19 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_17, x_18); x_20 = l_Lean_Json_mkObj(x_19); return x_20; } @@ -26262,7 +26262,7 @@ x_7 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_7, 0, x_6); lean_ctor_set(x_7, 1, x_5); x_8 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -26549,7 +26549,7 @@ x_17 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_17, 0, x_7); lean_ctor_set(x_17, 1, x_16); x_18 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_19 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_17, x_18); +x_19 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_17, x_18); x_20 = l_Lean_Json_mkObj(x_19); return x_20; } @@ -31072,7 +31072,7 @@ x_19 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_19, 0, x_10); lean_ctor_set(x_19, 1, x_18); x_20 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_21 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_19, x_20); +x_21 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_19, x_20); x_22 = l_Lean_Json_mkObj(x_21); return x_22; } @@ -31486,7 +31486,7 @@ x_20 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_20, 0, x_7); lean_ctor_set(x_20, 1, x_19); x_21 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_22 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_20, x_21); +x_22 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_20, x_21); x_23 = l_Lean_Json_mkObj(x_22); return x_23; } @@ -31655,7 +31655,7 @@ x_7 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_7, 0, x_6); lean_ctor_set(x_7, 1, x_5); x_8 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -31909,7 +31909,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_7); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -32405,7 +32405,7 @@ x_15 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_15, 0, x_4); lean_ctor_set(x_15, 1, x_14); x_16 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_17 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_15, x_16); +x_17 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_15, x_16); x_18 = l_Lean_Json_mkObj(x_17); return x_18; } @@ -32586,7 +32586,7 @@ x_7 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_7, 0, x_6); lean_ctor_set(x_7, 1, x_5); x_8 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -32859,7 +32859,7 @@ x_20 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_20, 0, x_8); lean_ctor_set(x_20, 1, x_19); x_21 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_22 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_20, x_21); +x_22 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_20, x_21); x_23 = l_Lean_Json_mkObj(x_22); return x_23; } @@ -33067,7 +33067,7 @@ x_7 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_7, 0, x_6); lean_ctor_set(x_7, 1, x_5); x_8 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -33444,7 +33444,7 @@ x_21 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_21, 0, x_8); lean_ctor_set(x_21, 1, x_20); x_22 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_23 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_21, x_22); +x_23 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_21, x_22); x_24 = l_Lean_Json_mkObj(x_23); return x_24; } @@ -33698,7 +33698,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_7); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } diff --git a/stage0/stdlib/Lean/Data/Lsp/TextSync.c b/stage0/stdlib/Lean/Data/Lsp/TextSync.c index b2f2f7517135..f9097fd91fdf 100644 --- a/stage0/stdlib/Lean/Data/Lsp/TextSync.c +++ b/stage0/stdlib/Lean/Data/Lsp/TextSync.c @@ -114,6 +114,7 @@ static lean_object* l___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_fromJsonTextD LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_toJsonDidChangeTextDocumentParams____x40_Lean_Data_Lsp_TextSync___hyg_529_(lean_object*); static lean_object* l_Lean_Lsp_instToJsonDidSaveTextDocumentParams___closed__1; static lean_object* l_Lean_Lsp_instFromJsonTextDocumentSyncKind___closed__3; +lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_fromJsonDidChangeTextDocumentParams____x40_Lean_Data_Lsp_TextSync___hyg_581____spec__1___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_fromJsonDidSaveTextDocumentParams____x40_Lean_Data_Lsp_TextSync___hyg_750____closed__11; static lean_object* l___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_fromJsonTextDocumentSyncOptions____x40_Lean_Data_Lsp_TextSync___hyg_1219____closed__19; @@ -127,7 +128,6 @@ static lean_object* l_Lean_Lsp_instFromJsonSaveOptions___closed__1; LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_fromJsonTextDocumentChangeRegistrationOptions____x40_Lean_Data_Lsp_TextSync___hyg_252____spec__1___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Lsp_instToJsonDidOpenTextDocumentParams___closed__1; static lean_object* l___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_fromJsonTextDocumentSyncOptions____x40_Lean_Data_Lsp_TextSync___hyg_1219____closed__18; -lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_fromJsonSaveOptions____x40_Lean_Data_Lsp_TextSync___hyg_906____closed__6; static lean_object* l___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_fromJsonSaveOptions____x40_Lean_Data_Lsp_TextSync___hyg_906____closed__3; static lean_object* l___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_fromJsonDidCloseTextDocumentParams____x40_Lean_Data_Lsp_TextSync___hyg_1023____closed__4; @@ -556,7 +556,7 @@ x_7 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_7, 0, x_6); lean_ctor_set(x_7, 1, x_5); x_8 = l___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_toJsonDidOpenTextDocumentParams____x40_Lean_Data_Lsp_TextSync___hyg_125____closed__2; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -1616,7 +1616,7 @@ x_17 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_17, 0, x_7); lean_ctor_set(x_17, 1, x_16); x_18 = l___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_toJsonDidOpenTextDocumentParams____x40_Lean_Data_Lsp_TextSync___hyg_125____closed__2; -x_19 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_17, x_18); +x_19 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_17, x_18); x_20 = l_Lean_Json_mkObj(x_19); return x_20; } @@ -2179,7 +2179,7 @@ x_12 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_12, 0, x_7); lean_ctor_set(x_12, 1, x_11); x_13 = l___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_toJsonDidOpenTextDocumentParams____x40_Lean_Data_Lsp_TextSync___hyg_125____closed__2; -x_14 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); +x_14 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); x_15 = l_Lean_Json_mkObj(x_14); return x_15; } @@ -2455,7 +2455,7 @@ x_7 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_7, 0, x_6); lean_ctor_set(x_7, 1, x_5); x_8 = l___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_toJsonDidOpenTextDocumentParams____x40_Lean_Data_Lsp_TextSync___hyg_125____closed__2; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -2655,7 +2655,7 @@ x_7 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_7, 0, x_6); lean_ctor_set(x_7, 1, x_5); x_8 = l___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_toJsonDidOpenTextDocumentParams____x40_Lean_Data_Lsp_TextSync___hyg_125____closed__2; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -3011,7 +3011,7 @@ x_27 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_27, 0, x_11); lean_ctor_set(x_27, 1, x_26); x_28 = l___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_toJsonDidOpenTextDocumentParams____x40_Lean_Data_Lsp_TextSync___hyg_125____closed__2; -x_29 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_27, x_28); +x_29 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_27, x_28); x_30 = l_Lean_Json_mkObj(x_29); return x_30; } @@ -3026,7 +3026,7 @@ x_33 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_33, 0, x_11); lean_ctor_set(x_33, 1, x_32); x_34 = l___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_toJsonDidOpenTextDocumentParams____x40_Lean_Data_Lsp_TextSync___hyg_125____closed__2; -x_35 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_33, x_34); +x_35 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_33, x_34); x_36 = l_Lean_Json_mkObj(x_35); return x_36; } @@ -3041,7 +3041,7 @@ x_39 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_39, 0, x_11); lean_ctor_set(x_39, 1, x_38); x_40 = l___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_toJsonDidOpenTextDocumentParams____x40_Lean_Data_Lsp_TextSync___hyg_125____closed__2; -x_41 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_39, x_40); +x_41 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_39, x_40); x_42 = l_Lean_Json_mkObj(x_41); return x_42; } diff --git a/stage0/stdlib/Lean/Data/Lsp/Window.c b/stage0/stdlib/Lean/Data/Lsp/Window.c index e323c52d2750..f1e8b38c7dde 100644 --- a/stage0/stdlib/Lean/Data/Lsp/Window.c +++ b/stage0/stdlib/Lean/Data/Lsp/Window.c @@ -47,7 +47,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_Window_0__fromJsonMessageActi static lean_object* l___private_Lean_Data_Lsp_Window_0__fromJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_134____closed__2; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_Window_0__toJsonShowMessageRequestParams____x40_Lean_Data_Lsp_Window___hyg_586_(lean_object*); static lean_object* l_instToJsonMessageType___closed__7; -LEAN_EXPORT lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_MessageType_toCtorIdx___boxed(lean_object*); static lean_object* l___private_Lean_Data_Lsp_Window_0__fromJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_134____closed__10; lean_object* lean_nat_to_int(lean_object*); @@ -137,6 +136,7 @@ static lean_object* l_instToJsonMessageType___closed__3; static lean_object* l___private_Lean_Data_Lsp_Window_0__fromJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_134____closed__13; static lean_object* l___private_Lean_Data_Lsp_Window_0__fromJsonShowMessageRequestParams____x40_Lean_Data_Lsp_Window___hyg_441____closed__8; static lean_object* l___private_Lean_Data_Lsp_Window_0__fromJsonShowMessageRequestParams____x40_Lean_Data_Lsp_Window___hyg_441____closed__14; +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(lean_object*, lean_object*); lean_object* l_Lean_Json_pretty(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_Window_0__fromJsonShowMessageRequestParams____x40_Lean_Data_Lsp_Window___hyg_441____closed__12; static lean_object* l___private_Lean_Data_Lsp_Window_0__fromJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_134____closed__12; @@ -1053,7 +1053,7 @@ x_1 = l_instFromJsonShowMessageParams___closed__1; return x_1; } } -LEAN_EXPORT lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -1211,7 +1211,7 @@ x_11 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_11, 0, x_10); lean_ctor_set(x_11, 1, x_9); x_12 = l___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____closed__1; -x_13 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_11, x_12); +x_13 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_11, x_12); x_14 = l_Lean_Json_mkObj(x_13); return x_14; } @@ -1223,7 +1223,7 @@ x_16 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_16, 0, x_15); lean_ctor_set(x_16, 1, x_9); x_17 = l___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____closed__1; -x_18 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_16, x_17); +x_18 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_16, x_17); x_19 = l_Lean_Json_mkObj(x_18); return x_19; } @@ -1235,7 +1235,7 @@ x_21 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_21, 0, x_20); lean_ctor_set(x_21, 1, x_9); x_22 = l___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____closed__1; -x_23 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_21, x_22); +x_23 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_21, x_22); x_24 = l_Lean_Json_mkObj(x_23); return x_24; } @@ -1247,7 +1247,7 @@ x_26 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_26, 0, x_25); lean_ctor_set(x_26, 1, x_9); x_27 = l___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____closed__1; -x_28 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_26, x_27); +x_28 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_26, x_27); x_29 = l_Lean_Json_mkObj(x_28); return x_29; } @@ -1456,7 +1456,7 @@ x_7 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_7, 0, x_6); lean_ctor_set(x_7, 1, x_5); x_8 = l___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____closed__1; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -2174,7 +2174,7 @@ x_15 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_15, 0, x_14); lean_ctor_set(x_15, 1, x_13); x_16 = l___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____closed__1; -x_17 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_15, x_16); +x_17 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_15, x_16); x_18 = l_Lean_Json_mkObj(x_17); return x_18; } @@ -2186,7 +2186,7 @@ x_20 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_20, 0, x_19); lean_ctor_set(x_20, 1, x_13); x_21 = l___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____closed__1; -x_22 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_20, x_21); +x_22 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_20, x_21); x_23 = l_Lean_Json_mkObj(x_22); return x_23; } @@ -2198,7 +2198,7 @@ x_25 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_25, 0, x_24); lean_ctor_set(x_25, 1, x_13); x_26 = l___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____closed__1; -x_27 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_25, x_26); +x_27 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_25, x_26); x_28 = l_Lean_Json_mkObj(x_27); return x_28; } @@ -2210,7 +2210,7 @@ x_30 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_30, 0, x_29); lean_ctor_set(x_30, 1, x_13); x_31 = l___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____closed__1; -x_32 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_30, x_31); +x_32 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_30, x_31); x_33 = l_Lean_Json_mkObj(x_32); return x_33; } diff --git a/stage0/stdlib/Lean/Data/Lsp/Workspace.c b/stage0/stdlib/Lean/Data/Lsp/Workspace.c index be035e77ffc9..8d0fdf23353b 100644 --- a/stage0/stdlib/Lean/Data/Lsp/Workspace.c +++ b/stage0/stdlib/Lean/Data/Lsp/Workspace.c @@ -101,6 +101,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_toJsonF static lean_object* l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_fromJsonDidChangeWatchedFilesRegistrationOptions____x40_Lean_Data_Lsp_Workspace___hyg_390____closed__5; static lean_object* l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_fromJsonDidChangeWatchedFilesRegistrationOptions____x40_Lean_Data_Lsp_Workspace___hyg_390____closed__2; static lean_object* l_Lean_Lsp_instFromJsonFileChangeType___closed__5; +lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_fromJsonDidChangeWatchedFilesRegistrationOptions____x40_Lean_Data_Lsp_Workspace___hyg_390____spec__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_fromJsonDidChangeWatchedFilesRegistrationOptions____x40_Lean_Data_Lsp_Workspace___hyg_390____spec__1___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_fromJsonFileEvent____x40_Lean_Data_Lsp_Workspace___hyg_640____closed__3; @@ -117,7 +118,6 @@ LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonFileEvent; static lean_object* l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_fromJsonFileEvent____x40_Lean_Data_Lsp_Workspace___hyg_640____closed__10; static lean_object* l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_fromJsonFileSystemWatcher____x40_Lean_Data_Lsp_Workspace___hyg_205____closed__10; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_toJsonDidChangeWatchedFilesRegistrationOptions____x40_Lean_Data_Lsp_Workspace___hyg_457____spec__1(size_t, size_t, lean_object*); -lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonFileEvent; static lean_object* l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_fromJsonDidChangeWatchedFilesRegistrationOptions____x40_Lean_Data_Lsp_Workspace___hyg_390____closed__1; static lean_object* l_Lean_Lsp_instToJsonFileSystemWatcher___closed__1; @@ -242,7 +242,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_8); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_toJsonWorkspaceFolder____x40_Lean_Data_Lsp_Workspace___hyg_25____closed__3; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -280,7 +280,7 @@ x_30 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_30, 0, x_24); lean_ctor_set(x_30, 1, x_29); x_31 = l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_toJsonWorkspaceFolder____x40_Lean_Data_Lsp_Workspace___hyg_25____closed__3; -x_32 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_30, x_31); +x_32 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_30, x_31); x_33 = l_Lean_Json_mkObj(x_32); return x_33; } @@ -923,7 +923,7 @@ x_10 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_10, 0, x_8); lean_ctor_set(x_10, 1, x_9); x_11 = l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_toJsonWorkspaceFolder____x40_Lean_Data_Lsp_Workspace___hyg_25____closed__3; -x_12 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_10, x_11); +x_12 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_10, x_11); x_13 = l_Lean_Json_mkObj(x_12); return x_13; } @@ -952,7 +952,7 @@ x_21 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_21, 0, x_8); lean_ctor_set(x_21, 1, x_20); x_22 = l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_toJsonWorkspaceFolder____x40_Lean_Data_Lsp_Workspace___hyg_25____closed__3; -x_23 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_21, x_22); +x_23 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_21, x_22); x_24 = l_Lean_Json_mkObj(x_23); return x_24; } @@ -979,7 +979,7 @@ x_32 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_32, 0, x_8); lean_ctor_set(x_32, 1, x_31); x_33 = l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_toJsonWorkspaceFolder____x40_Lean_Data_Lsp_Workspace___hyg_25____closed__3; -x_34 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_32, x_33); +x_34 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_32, x_33); x_35 = l_Lean_Json_mkObj(x_34); return x_35; } @@ -1011,7 +1011,7 @@ x_44 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_44, 0, x_42); lean_ctor_set(x_44, 1, x_43); x_45 = l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_toJsonWorkspaceFolder____x40_Lean_Data_Lsp_Workspace___hyg_25____closed__3; -x_46 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_44, x_45); +x_46 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_44, x_45); x_47 = l_Lean_Json_mkObj(x_46); return x_47; } @@ -1049,7 +1049,7 @@ x_56 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_56, 0, x_42); lean_ctor_set(x_56, 1, x_55); x_57 = l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_toJsonWorkspaceFolder____x40_Lean_Data_Lsp_Workspace___hyg_25____closed__3; -x_58 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_56, x_57); +x_58 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_56, x_57); x_59 = l_Lean_Json_mkObj(x_58); return x_59; } @@ -1477,7 +1477,7 @@ x_10 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_10, 0, x_9); lean_ctor_set(x_10, 1, x_8); x_11 = l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_toJsonWorkspaceFolder____x40_Lean_Data_Lsp_Workspace___hyg_25____closed__3; -x_12 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_10, x_11); +x_12 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_10, x_11); x_13 = l_Lean_Json_mkObj(x_12); return x_13; } @@ -2419,7 +2419,7 @@ x_10 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_10, 0, x_8); lean_ctor_set(x_10, 1, x_9); x_11 = l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_toJsonWorkspaceFolder____x40_Lean_Data_Lsp_Workspace___hyg_25____closed__3; -x_12 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_10, x_11); +x_12 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_10, x_11); x_13 = l_Lean_Json_mkObj(x_12); return x_13; } @@ -2431,7 +2431,7 @@ x_15 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_15, 0, x_8); lean_ctor_set(x_15, 1, x_14); x_16 = l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_toJsonWorkspaceFolder____x40_Lean_Data_Lsp_Workspace___hyg_25____closed__3; -x_17 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_15, x_16); +x_17 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_15, x_16); x_18 = l_Lean_Json_mkObj(x_17); return x_18; } @@ -2443,7 +2443,7 @@ x_20 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_20, 0, x_8); lean_ctor_set(x_20, 1, x_19); x_21 = l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_toJsonWorkspaceFolder____x40_Lean_Data_Lsp_Workspace___hyg_25____closed__3; -x_22 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_20, x_21); +x_22 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_20, x_21); x_23 = l_Lean_Json_mkObj(x_22); return x_23; } @@ -2841,7 +2841,7 @@ x_10 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_10, 0, x_9); lean_ctor_set(x_10, 1, x_8); x_11 = l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_toJsonWorkspaceFolder____x40_Lean_Data_Lsp_Workspace___hyg_25____closed__3; -x_12 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_10, x_11); +x_12 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_10, x_11); x_13 = l_Lean_Json_mkObj(x_12); return x_13; } diff --git a/stage0/stdlib/Lean/Data/Position.c b/stage0/stdlib/Lean/Data/Position.c index 0e01c7ea27c2..3faad395f081 100644 --- a/stage0/stdlib/Lean/Data/Position.c +++ b/stage0/stdlib/Lean/Data/Position.c @@ -138,8 +138,8 @@ lean_object* lean_array_get_size(lean_object*); static lean_object* l___private_Lean_Data_Position_0__Lean_fromJsonPosition____x40_Lean_Data_Position___hyg_289____closed__3; uint8_t lean_nat_dec_le(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_Position_0__Lean_decEqPosition____x40_Lean_Data_Position___hyg_34____boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_bindTR_go___at___private_Lean_Data_Position_0__Lean_toJsonPosition____x40_Lean_Data_Position___hyg_237____spec__1(lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Position_0__Lean_toJsonPosition____x40_Lean_Data_Position___hyg_237____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_Position_0__Lean_toJsonPosition____x40_Lean_Data_Position___hyg_237_(lean_object*); static lean_object* l_Lean_Position_instToFormat___closed__6; LEAN_EXPORT lean_object* l_Lean_FileMap_toPosition_loop(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -488,7 +488,7 @@ x_1 = l_Lean_instReprPosition___closed__1; return x_1; } } -LEAN_EXPORT lean_object* l_List_bindTR_go___at___private_Lean_Data_Position_0__Lean_toJsonPosition____x40_Lean_Data_Position___hyg_237____spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Position_0__Lean_toJsonPosition____x40_Lean_Data_Position___hyg_237____spec__1(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -558,7 +558,7 @@ x_16 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_16, 0, x_8); lean_ctor_set(x_16, 1, x_15); x_17 = l___private_Lean_Data_Position_0__Lean_toJsonPosition____x40_Lean_Data_Position___hyg_237____closed__1; -x_18 = l_List_bindTR_go___at___private_Lean_Data_Position_0__Lean_toJsonPosition____x40_Lean_Data_Position___hyg_237____spec__1(x_16, x_17); +x_18 = l_List_flatMapTR_go___at___private_Lean_Data_Position_0__Lean_toJsonPosition____x40_Lean_Data_Position___hyg_237____spec__1(x_16, x_17); x_19 = l_Lean_Json_mkObj(x_18); return x_19; } diff --git a/stage0/stdlib/Lean/Data/Trie.c b/stage0/stdlib/Lean/Data/Trie.c index 48f8d680db1a..51de47874c7e 100644 --- a/stage0/stdlib/Lean/Data/Trie.c +++ b/stage0/stdlib/Lean/Data/Trie.c @@ -61,6 +61,7 @@ LEAN_EXPORT lean_object* l_Lean_Data_Trie_findPrefix_go___rarg(lean_object*, lea LEAN_EXPORT lean_object* l_Lean_Data_Trie_matchPrefix_loop___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Data_Trie_values_go___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Data_Trie_instEmptyCollection(lean_object*); +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Trie_0__Lean_Data_Trie_toStringAux___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Data_Trie_matchPrefix_loop___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Data_Trie_upsert_loop___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Data_Trie_matchPrefix_loop(lean_object*); @@ -81,7 +82,6 @@ LEAN_EXPORT lean_object* l_ByteArray_findIdx_x3f_loop___at_Lean_Data_Trie_matchP LEAN_EXPORT lean_object* l_Lean_Data_Trie_upsert___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Data_Trie_insert___rarg___lambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Data_Trie_upsert_loop___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_bindTR_go___at___private_Lean_Data_Trie_0__Lean_Data_Trie_toStringAux___spec__1(lean_object*, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Data_Trie_values_go___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Data_Trie_upsert(lean_object*); @@ -1769,7 +1769,7 @@ lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_List_bindTR_go___at___private_Lean_Data_Trie_0__Lean_Data_Trie_toStringAux___spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Trie_0__Lean_Data_Trie_toStringAux___spec__1(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -1895,7 +1895,7 @@ x_21 = lean_array_to_list(x_19); x_22 = l___private_Lean_Data_Trie_0__Lean_Data_Trie_toStringAux___rarg___closed__1; x_23 = l_Lean_Data_Trie_values___rarg___closed__1; x_24 = l_List_zipWithTR_go___rarg(x_22, x_20, x_21, x_23); -x_25 = l_List_bindTR_go___at___private_Lean_Data_Trie_0__Lean_Data_Trie_toStringAux___spec__1(x_24, x_23); +x_25 = l_List_flatMapTR_go___at___private_Lean_Data_Trie_0__Lean_Data_Trie_toStringAux___spec__1(x_24, x_23); return x_25; } } diff --git a/stage0/stdlib/Lean/Declaration.c b/stage0/stdlib/Lean/Declaration.c index b05ffad0183b..0eae7f9dc0a0 100644 --- a/stage0/stdlib/Lean/Declaration.c +++ b/stage0/stdlib/Lean/Declaration.c @@ -38,15 +38,18 @@ LEAN_EXPORT lean_object* l_Lean_ConstantInfo_levelParams(lean_object*); LEAN_EXPORT lean_object* l_Lean_Declaration_foldExprM___at_Lean_Declaration_forExprM___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Declaration_definitionVal_x21___boxed(lean_object*); static lean_object* l___private_Lean_Declaration_0__Lean_reprDefinitionSafety____x40_Lean_Declaration___hyg_685____closed__3; +LEAN_EXPORT lean_object* l_Lean_RecursorVal_getMajorInduct_go(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_instBEqConstantVal; LEAN_EXPORT lean_object* l_Lean_mkAxiomValEx___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_instInhabitedRecursorVal___closed__1; static lean_object* l_Lean_instReprDefinitionSafety___closed__1; LEAN_EXPORT lean_object* l_Lean_Declaration_isUnsafeInductiveDeclEx___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Lean_RecursorVal_getMajorInduct(lean_object*); LEAN_EXPORT lean_object* l_Lean_ConstantInfo_inductiveVal_x21(lean_object*); LEAN_EXPORT uint8_t l_List_beq___at___private_Lean_Declaration_0__Lean_beqRecursorVal____x40_Lean_Declaration___hyg_3174____spec__1(lean_object*, lean_object*); static lean_object* l_Lean_instInhabitedDeclaration___closed__1; LEAN_EXPORT lean_object* l_Lean_mkRecursorValEx___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_ConstantInfo_isTheorem___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_instInhabitedTheoremVal; LEAN_EXPORT lean_object* lean_mk_reducibility_hints_regular(uint32_t); lean_object* l_List_foldlM___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -104,6 +107,7 @@ static lean_object* l___private_Lean_Declaration_0__Lean_reprDefinitionSafety___ LEAN_EXPORT lean_object* l_Lean_instBEqDefinitionSafety; LEAN_EXPORT lean_object* l_Lean_DefinitionSafety_toCtorIdx___boxed(lean_object*); static lean_object* l___private_Lean_Declaration_0__Lean_reprDefinitionSafety____x40_Lean_Declaration___hyg_685____closed__12; +LEAN_EXPORT uint8_t l_Lean_ConstantInfo_isTheorem(lean_object*); static lean_object* l_Lean_instInhabitedConstructorVal___closed__1; LEAN_EXPORT lean_object* l_Lean_instBEqAxiomVal; static lean_object* l_Lean_instInhabitedConstantInfo___closed__1; @@ -123,7 +127,6 @@ LEAN_EXPORT uint8_t l___private_Lean_Declaration_0__Lean_beqDeclaration____x40_L LEAN_EXPORT lean_object* l_Lean_Declaration_foldExprM___at_Lean_Declaration_forExprM___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_instBEqInductiveType; static lean_object* l_Lean_ConstantInfo_value_x21___closed__3; -lean_object* l_Lean_Name_getPrefix(lean_object*); LEAN_EXPORT uint8_t l_Lean_ConstantInfo_isCtor(lean_object*); LEAN_EXPORT lean_object* l_List_foldlM___at_Lean_Declaration_forExprM___spec__2___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_instInhabitedConstantVal___closed__2; @@ -156,6 +159,7 @@ static lean_object* l___private_Lean_Declaration_0__Lean_reprDefinitionSafety___ LEAN_EXPORT uint8_t l_List_beq___at___private_Lean_Declaration_0__Lean_beqDeclaration____x40_Lean_Declaration___hyg_1774____spec__2(lean_object*, lean_object*); LEAN_EXPORT uint8_t lean_axiom_val_is_unsafe(lean_object*); LEAN_EXPORT uint32_t lean_reducibility_hints_get_height(lean_object*); +lean_object* l_Lean_Expr_constName_x21(lean_object*); static lean_object* l___private_Lean_Declaration_0__Lean_reprDefinitionSafety____x40_Lean_Declaration___hyg_685____closed__18; LEAN_EXPORT lean_object* l_Lean_instInhabitedConstructor; LEAN_EXPORT lean_object* l_Lean_ConstantInfo_numLevelParams___boxed(lean_object*); @@ -182,7 +186,6 @@ LEAN_EXPORT uint8_t l_Lean_instInhabitedDefinitionSafety; static lean_object* l___private_Lean_Declaration_0__Lean_reprDefinitionSafety____x40_Lean_Declaration___hyg_685____closed__7; LEAN_EXPORT lean_object* l_Lean_instBEqDeclaration; LEAN_EXPORT lean_object* l_Lean_DefinitionSafety_noConfusion___rarg(uint8_t, uint8_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_RecursorVal_getInduct(lean_object*); LEAN_EXPORT lean_object* l_Lean_Declaration_foldExprM___rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ReducibilityHints_lt___boxed(lean_object*, lean_object*); LEAN_EXPORT uint8_t lean_recursor_k(lean_object*); @@ -205,6 +208,7 @@ static lean_object* l_Lean_instBEqReducibilityHints___closed__1; static lean_object* l_Lean_ReducibilityHints_instOrd___closed__1; LEAN_EXPORT uint8_t lean_is_unsafe_inductive_decl(lean_object*); LEAN_EXPORT lean_object* l_List_beq___at___private_Lean_Declaration_0__Lean_beqConstantVal____x40_Lean_Declaration___hyg_433____spec__1___boxed(lean_object*, lean_object*); +lean_object* l_Lean_Expr_bindingDomain_x21(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Declaration_0__Lean_reprDefinitionSafety____x40_Lean_Declaration___hyg_685_(uint8_t, lean_object*); LEAN_EXPORT uint8_t lean_inductive_val_is_reflexive(lean_object*); LEAN_EXPORT lean_object* l_List_foldlM___at_Lean_Declaration_forExprM___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*); @@ -237,8 +241,10 @@ LEAN_EXPORT lean_object* l___private_Lean_Declaration_0__Lean_beqDefinitionVal__ lean_object* l_Repr_addAppParen(lean_object*, lean_object*); lean_object* lean_panic_fn(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_ReducibilityHints_isAbbrev(lean_object*); +lean_object* lean_nat_sub(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_InductiveVal_isNested___boxed(lean_object*); static lean_object* l_Lean_instBEqTheoremVal___closed__1; +lean_object* l_Lean_Expr_getAppFn(lean_object*); static lean_object* l___private_Lean_Declaration_0__Lean_reprDefinitionSafety____x40_Lean_Declaration___hyg_685____closed__14; static lean_object* l_Lean_instInhabitedInductiveType___closed__1; LEAN_EXPORT uint8_t l___private_Lean_Declaration_0__Lean_beqRecursorRule____x40_Lean_Declaration___hyg_2988_(lean_object*, lean_object*); @@ -256,7 +262,6 @@ static lean_object* l_Lean_instInhabitedDefinitionVal___closed__1; LEAN_EXPORT lean_object* l_Lean_instInhabitedOpaqueVal; uint8_t lean_uint32_dec_lt(uint32_t, uint32_t); LEAN_EXPORT uint8_t l___private_Lean_Declaration_0__Lean_beqDefinitionSafety____x40_Lean_Declaration___hyg_667_(uint8_t, uint8_t); -LEAN_EXPORT lean_object* l_Lean_RecursorVal_getInduct___boxed(lean_object*); static lean_object* l_Lean_instBEqOpaqueVal___closed__1; LEAN_EXPORT lean_object* l_Lean_instInhabitedDefinitionVal; LEAN_EXPORT uint8_t l___private_Lean_Declaration_0__Lean_beqRecursorVal____x40_Lean_Declaration___hyg_3174_(lean_object*, lean_object*); @@ -267,6 +272,7 @@ LEAN_EXPORT lean_object* l_Lean_RecursorVal_getFirstMinorIdx___boxed(lean_object LEAN_EXPORT lean_object* l_Lean_ConstantInfo_levelParams___boxed(lean_object*); static lean_object* l_Lean_Declaration_definitionVal_x21___closed__3; static lean_object* l_Lean_Declaration_definitionVal_x21___closed__4; +lean_object* l_Lean_Expr_bindingBody_x21(lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Declaration_0__Lean_beqReducibilityHints____x40_Lean_Declaration___hyg_27_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_DefinitionSafety_noConfusion___rarg___lambda__1___boxed(lean_object*); static lean_object* l_Lean_instInhabitedRecursorRule___closed__1; @@ -3888,23 +3894,51 @@ lean_dec(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_RecursorVal_getInduct(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_RecursorVal_getMajorInduct_go(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_2 = lean_ctor_get(x_1, 0); -x_3 = lean_ctor_get(x_2, 0); -x_4 = l_Lean_Name_getPrefix(x_3); -return x_4; +lean_object* x_3; uint8_t x_4; +x_3 = lean_unsigned_to_nat(0u); +x_4 = lean_nat_dec_eq(x_1, x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_5 = lean_unsigned_to_nat(1u); +x_6 = lean_nat_sub(x_1, x_5); +lean_dec(x_1); +x_7 = l_Lean_Expr_bindingBody_x21(x_2); +lean_dec(x_2); +x_1 = x_6; +x_2 = x_7; +goto _start; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; +lean_dec(x_1); +x_9 = l_Lean_Expr_bindingDomain_x21(x_2); +lean_dec(x_2); +x_10 = l_Lean_Expr_getAppFn(x_9); +lean_dec(x_9); +x_11 = l_Lean_Expr_constName_x21(x_10); +lean_dec(x_10); +return x_11; } } -LEAN_EXPORT lean_object* l_Lean_RecursorVal_getInduct___boxed(lean_object* x_1) { +} +LEAN_EXPORT lean_object* l_Lean_RecursorVal_getMajorInduct(lean_object* x_1) { _start: { -lean_object* x_2; -x_2 = l_Lean_RecursorVal_getInduct(x_1); +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_2 = l_Lean_RecursorVal_getMajorIdx(x_1); +x_3 = lean_ctor_get(x_1, 0); +lean_inc(x_3); lean_dec(x_1); -return x_2; +x_4 = lean_ctor_get(x_3, 2); +lean_inc(x_4); +lean_dec(x_3); +x_5 = l_Lean_RecursorVal_getMajorInduct_go(x_2, x_4); +return x_5; } } LEAN_EXPORT lean_object* l_Lean_QuotKind_toCtorIdx(uint8_t x_1) { @@ -4388,7 +4422,7 @@ static lean_object* _init_l_Lean_ConstantInfo_value_x21___closed__3() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Declaration_definitionVal_x21___closed__1; x_2 = l_Lean_ConstantInfo_value_x21___closed__1; -x_3 = lean_unsigned_to_nat(456u); +x_3 = lean_unsigned_to_nat(461u); x_4 = lean_unsigned_to_nat(33u); x_5 = l_Lean_ConstantInfo_value_x21___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -4516,6 +4550,33 @@ x_3 = lean_box(x_2); return x_3; } } +LEAN_EXPORT uint8_t l_Lean_ConstantInfo_isTheorem(lean_object* x_1) { +_start: +{ +if (lean_obj_tag(x_1) == 2) +{ +uint8_t x_2; +x_2 = 1; +return x_2; +} +else +{ +uint8_t x_3; +x_3 = 0; +return x_3; +} +} +} +LEAN_EXPORT lean_object* l_Lean_ConstantInfo_isTheorem___boxed(lean_object* x_1) { +_start: +{ +uint8_t x_2; lean_object* x_3; +x_2 = l_Lean_ConstantInfo_isTheorem(x_1); +lean_dec(x_1); +x_3 = lean_box(x_2); +return x_3; +} +} LEAN_EXPORT lean_object* l_panic___at_Lean_ConstantInfo_inductiveVal_x21___spec__1(lean_object* x_1) { _start: { @@ -4547,7 +4608,7 @@ static lean_object* _init_l_Lean_ConstantInfo_inductiveVal_x21___closed__3() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Declaration_definitionVal_x21___closed__1; x_2 = l_Lean_ConstantInfo_inductiveVal_x21___closed__1; -x_3 = lean_unsigned_to_nat(472u); +x_3 = lean_unsigned_to_nat(481u); x_4 = lean_unsigned_to_nat(9u); x_5 = l_Lean_ConstantInfo_inductiveVal_x21___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Elab/App.c b/stage0/stdlib/Lean/Elab/App.c index 6bdd5849103f..181ffcc9555f 100644 --- a/stage0/stdlib/Lean/Elab/App.c +++ b/stage0/stdlib/Lean/Elab/App.c @@ -220,7 +220,6 @@ static lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveLValAux__ LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_shouldElabAsElim___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_findNamedArgDependsOnCurrent_x3f___spec__4(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_findField_x3f(lean_object*, lean_object*, lean_object*); -uint8_t l_Array_contains___at_Lean_findField_x3f___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_ElabElim_mkMotive(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_resolveLValAux___closed__2; static lean_object* l_Lean_Elab_Term_ElabElim_finalize___closed__1; @@ -1102,6 +1101,7 @@ static lean_object* l_Lean_Elab_Term_ElabElim_finalize___lambda__9___closed__6; LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_addLValArg_go___lambda__1(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*); static lean_object* l_Lean_Elab_Term_getElabElimExprInfo___closed__3; +uint8_t l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_ElabElim_finalize___lambda__5___boxed(lean_object**); static lean_object* l_Lean_Elab_Term_ElabElim_finalize___lambda__9___closed__8; lean_object* l_Lean_LocalDecl_type(lean_object*); @@ -44274,7 +44274,7 @@ lean_dec(x_67); x_68 = lean_ctor_get(x_58, 0); lean_inc(x_68); lean_dec(x_58); -x_69 = l_Array_contains___at_Lean_findField_x3f___spec__1(x_37, x_68); +x_69 = l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(x_37, x_68); if (x_69 == 0) { lean_object* x_70; lean_object* x_71; uint8_t x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; @@ -44807,7 +44807,7 @@ lean_dec(x_182); x_183 = lean_ctor_get(x_173, 0); lean_inc(x_183); lean_dec(x_173); -x_184 = l_Array_contains___at_Lean_findField_x3f___spec__1(x_37, x_183); +x_184 = l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(x_37, x_183); if (x_184 == 0) { lean_object* x_185; lean_object* x_186; uint8_t 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; diff --git a/stage0/stdlib/Lean/Elab/BuiltinCommand.c b/stage0/stdlib/Lean/Elab/BuiltinCommand.c index 012a45bc3678..25141ae3ea33 100644 --- a/stage0/stdlib/Lean/Elab/BuiltinCommand.c +++ b/stage0/stdlib/Lean/Elab/BuiltinCommand.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Lean.Elab.BuiltinCommand -// Imports: Lean.Util.CollectLevelParams Lean.Util.CollectAxioms Lean.Meta.Reduce Lean.Elab.DeclarationRange Lean.Elab.Eval Lean.Elab.Command Lean.Elab.Open Lean.Elab.SetOption +// Imports: Lean.Util.CollectLevelParams Lean.Util.CollectAxioms Lean.Meta.Reduce Lean.Elab.DeclarationRange Lean.Elab.Eval Lean.Elab.Command Lean.Elab.Open Lean.Elab.SetOption Init.System.Platform #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -19,21 +19,22 @@ lean_object* l_Lean_Name_getNumParts(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabReduce__1___closed__1; static lean_object* l_Lean_getDocStringText___at_Lean_Elab_Command_elabAddDeclDoc___spec__2___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Command_elabUniverse__1___closed__5; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabExport___spec__23(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabReduce__1___closed__2; static lean_object* l_Lean_Elab_Command_elabOmit___closed__1; lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); lean_object* lean_string_utf8_extract(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___closed__2; +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__24; lean_object* l_Lean_Elab_Term_levelMVarToParam(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabCheckFailure_declRange__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabExport(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__11___closed__1; LEAN_EXPORT lean_object* l_Lean_Syntax_forArgsM___at_Lean_Elab_Command_elabUniverse___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabUniverse___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabReduce_declRange__1___closed__5; -LEAN_EXPORT lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__1; +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__19; static lean_object* l___regBuiltin_Lean_Elab_Command_elabCheck__1___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Command_elabAddDeclDoc_declRange__1___closed__7; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Elab_Command_elabOmit___spec__10___boxed(lean_object*, lean_object*); @@ -52,39 +53,41 @@ static lean_object* l_Lean_Elab_Command_elabEnd___lambda__1___closed__9; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabOmit(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabExit_declRange__1___closed__4; lean_object* l_Lean_MapDeclarationExtension_insert___rarg(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__7___closed__3; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabChoice___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___lambda__1(lean_object*, lean_object*, uint8_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabSection__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabVersion___boxed(lean_object*); lean_object* l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_mkConstWithLevelParams___at_Lean_Elab_Command_elabOpen___spec__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__4; lean_object* l_Lean_Elab_addCompletionInfo___at_Lean_withSetOptionIn___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getDocStringText___at_Lean_Elab_Command_elabAddDeclDoc___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_hasNoErrorMessages___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabVersion(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabNamespace_declRange__1___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Command_elabChoice__1___closed__1; lean_object* l_Array_sequenceMap___at_Lean_Elab_OpenDecl_elabOpenDecl___spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabSetOption__1(lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabExport___spec__24___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabCheck_declRange__1___closed__4; lean_object* l_Lean_ScopedEnvExtension_activateScoped___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_OpenDecl_resolveId___at_Lean_Elab_Command_elabExport___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOpen___spec__23___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabSection_declRange__1___closed__5; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabOpen___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Command_elabEnd_declRange__1___closed__2; +static lean_object* l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_addScope___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_OpenDecl_resolveId___at_Lean_Elab_Command_elabExport___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_hasNoErrorMessages(lean_object*); -static lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__11___closed__2; LEAN_EXPORT lean_object* l_Lean_popScope___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_popScopes___spec__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabChoice_declRange__1___closed__1; static lean_object* l_Lean_Elab_Command_failIfSucceeds___closed__2; static lean_object* l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_elabOpen___spec__15___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Command_elabInitQuot_declRange__1___closed__3; LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabExport___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__14___closed__2; lean_object* l_Lean_Elab_Command_runTermElabM___rarg(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*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabModuleDoc_declRange__1___closed__6; @@ -92,8 +95,8 @@ LEAN_EXPORT lean_object* l_Lean_setEnv___at_Lean_Elab_Command_elabInitQuot___spe static lean_object* l_Lean_Elab_Command_elabReduce_go___lambda__1___closed__2; static lean_object* l_List_forIn_loop___at_Lean_Elab_Command_elabCheckCore___spec__1___closed__5; extern lean_object* l_Lean_declRangeExt; -static lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___lambda__1___closed__1; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_addDocString___at_Lean_Elab_Command_elabAddDeclDoc___spec__5___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5(uint8_t, lean_object*, uint8_t, 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_Command_elabOpen___spec__19(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabCheckFailure__1___closed__1; static lean_object* l_Lean_Elab_Command_elabSetOption___closed__1; @@ -102,6 +105,7 @@ static lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_ty static lean_object* l_Lean_Elab_Command_elabAddDeclDoc___closed__5; static lean_object* l_Lean_Elab_Command_expandInCmd___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOpen___spec__17(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__17; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabVariable___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabExit__1___closed__5; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabVariable___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -112,8 +116,9 @@ LEAN_EXPORT lean_object* l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elab lean_object* l_Lean_indentD(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabModuleDoc__1___closed__6; static lean_object* l_Lean_Elab_Command_elabExit___rarg___closed__2; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___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_addConstInfo___at_Lean_Elab_Command_elabOpen___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__2; +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__30; uint8_t l_Lean_Exception_isInterrupt(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabExit__1___closed__4; LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabAddDeclDoc___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -121,32 +126,32 @@ lean_object* l_Lean_Elab_Command_getMainModule___rarg(lean_object*, lean_object* lean_object* l_Lean_Elab_Term_synthesizeSyntheticMVars(uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabEoi__1___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabCheck__1(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_addConstInfo___at_Lean_Elab_Command_elabExport___spec__22___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__16; lean_object* l_Lean_Elab_Term_elabTerm(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_pushScope___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_addScope___spec__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabReduce_go___lambda__1(lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_isExprDefEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__15; lean_object* l_Lean_FileMap_toPosition(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabImport___rarg___closed__1; static lean_object* l_Lean_Elab_Command_elabOmit___lambda__1___closed__1; -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabExport___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__5___closed__4; LEAN_EXPORT lean_object* l_Lean_Syntax_forArgsM___at_Lean_Elab_Command_elabUniverse___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_uint64_to_usize(uint64_t); static lean_object* l___regBuiltin_Lean_Elab_Command_elabSection__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabNamespace___spec__1(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__34; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Command_elabOpen___spec__24___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInclude___spec__1___lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabOpen___spec__14(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_addCompletionInfo___at_Lean_Elab_Term_addDotCompletionInfo___spec__1(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_Command_elabCommand___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_toString(lean_object*, uint8_t, lean_object*); -lean_object* l_Lean_addDocString___at_Lean_Elab_Command_expandDeclId___spec__14(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_containsId___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getId(lean_object*); uint8_t l_List_beq___at___private_Lean_Data_OpenDecl_0__Lean_beqOpenDecl____x40_Lean_Data_OpenDecl___hyg_40____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInitQuot___boxed(lean_object*); +extern uint8_t l_System_Platform_isOSX; static lean_object* l___regBuiltin_Lean_Elab_Command_expandInCmd__1___closed__4; lean_object* l_Array_findIdx_x3f_loop___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabModuleDoc__1(lean_object*); @@ -154,32 +159,36 @@ lean_object* l_Lean_MessageData_ofList(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabEnd__1___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Command_elabExit__1___closed__1; lean_object* l_Lean_PersistentArray_push___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabCheckFailure__1(lean_object*); static lean_object* l_Lean_Elab_Command_elabReduce___closed__1; lean_object* l_Array_toSubarray___rarg(lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__3___closed__2; LEAN_EXPORT uint8_t l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInclude___spec__1___lambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabExit___boxed(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabModuleDoc__1___closed__3; -uint8_t l_Array_contains___at_Lean_findField_x3f___spec__1(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__10; +lean_object* l_String_removeLeadingSpaces(lean_object*); static lean_object* l_Lean_Elab_Command_elabCheckFailure___closed__3; -static lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___closed__1; LEAN_EXPORT lean_object* l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabOpen___spec__7(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabVariable___closed__2; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Elab_Command_elabOmit___spec__8(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabSynth__1___closed__2; lean_object* lean_mk_array(lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); +LEAN_EXPORT lean_object* l_Lean_filterFieldList___at_Lean_Elab_Command_elabExport___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_failIfSucceeds___lambda__1(uint8_t, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabExit___rarg___closed__1; +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabUniverse_declRange__1___closed__3; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabExport___spec__28___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getArgs(lean_object*); -LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAddDeclDoc___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___closed__2; LEAN_EXPORT lean_object* l_Lean_mkConstWithLevelParams___at_Lean_Elab_Command_elabOpen___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabOpen_declRange__1___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Command_elabCheckFailure_declRange__1___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Command_elabInitQuot_declRange__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabInclude__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabReduce_go(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_replaceRef(lean_object*, lean_object*); @@ -187,6 +196,8 @@ static lean_object* l___regBuiltin_Lean_Elab_Command_elabNamespace_declRange__1_ LEAN_EXPORT lean_object* l_Lean_Syntax_foldArgsM___at_Lean_Elab_Command_elabUniverse___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabOpen_declRange__1___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_addScopes(uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_addDocString___at_Lean_Elab_Command_elabAddDeclDoc___spec__5___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabReduce_go___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__5___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*); @@ -195,12 +206,10 @@ lean_object* l_Lean_Elab_Command_elabCommand(lean_object*, lean_object*, lean_ob lean_object* lean_array_fget(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_popScopes(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabUniverse__1___closed__3; +static lean_object* l_Lean_addDocString___at_Lean_Elab_Command_elabAddDeclDoc___spec__5___closed__2; lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabExport___spec__21(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabImport_declRange__1___closed__3; -lean_object* l_Lean_Syntax_getTailPos_x3f(lean_object*, uint8_t); static lean_object* l_Lean_Elab_Command_elabReduce_go___lambda__1___closed__1; -lean_object* l_Lean_mkConstWithLevelParams___at_Lean_Elab_Command_expandDeclId___spec__8(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Command_getScopes___rarg(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabExport_declRange__1___closed__6; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabVariable___spec__2___at_Lean_Elab_Command_elabVariable___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -209,24 +218,31 @@ static lean_object* l_Lean_Elab_Command_elabEnd___lambda__1___closed__7; static lean_object* l_Lean_logWarning___at_Lean_Elab_Command_elabExit___spec__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabReduce_go___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabOmit___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__14; +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__11; lean_object* l_Lean_Expr_fvarId_x21(lean_object*); extern lean_object* l_Lean_instInhabitedException; static lean_object* l___regBuiltin_Lean_Elab_Command_expandInCmd__1___closed__3; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__5; +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__18; lean_object* l_Lean_ScopedEnvExtension_pushScope___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabVariable_declRange__1(lean_object*); lean_object* lean_environment_find(lean_object*, lean_object*); lean_object* l_Lean_Elab_Command_addUnivLevel___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_getRefPos___at_Lean_Elab_Command_elabExport___spec__21___boxed(lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_expandInCmd__1(lean_object*); +LEAN_EXPORT lean_object* l_Lean_getRefPos___at_Lean_Elab_Command_elabExport___spec__21___rarg___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_filterFieldList___at_Lean_Elab_Command_elabExport___spec__11___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabOpen___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSection___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabChoice(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_filterFieldList___at_Lean_Elab_Command_elabExport___spec__10___lambda__1(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 uint8_t l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___lambda__2(lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabReduce__1(lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___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_BuiltinCommand_0__Lean_Elab_Command_addScope___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOpen___spec__17___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_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabNonComputableSection___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_foldArgsM___at_Lean_Elab_Command_elabUniverse___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_findDeclarationRangesCore_x3f___at_Lean_Elab_Command_elabAddDeclDoc___spec__1___closed__1; @@ -236,21 +252,21 @@ lean_object* l_Lean_Syntax_node5(lean_object*, lean_object*, lean_object*, lean_ static lean_object* l___regBuiltin_Lean_Elab_Command_elabReduce_declRange__1___closed__4; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabExport__1(lean_object*); uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__39; lean_object* l_Nat_nextPowerOfTwo_go(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabSetOption_declRange__1(lean_object*); -static lean_object* l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Command_elabAddDeclDoc_declRange__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabEnd(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabCheckFailure__1___closed__2; lean_object* l_Lean_stringToMessageData(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabSetOption_declRange__1___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Command_expandInCmd_declRange__1___closed__4; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6___closed__3; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_popScopes___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabNamespace_declRange__1(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___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_Elab_Command_elabCheckCore___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___regBuiltin_Lean_Elab_Command_elabModuleDoc_declRange__1___closed__1; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__1; +LEAN_EXPORT lean_object* l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabSetOption__1___closed__4; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabNonComputableSection_declRange__1(lean_object*); uint8_t l_Lean_MapDeclarationExtension_contains___rarg(lean_object*, lean_object*, lean_object*, lean_object*); @@ -263,25 +279,30 @@ static lean_object* l___regBuiltin_Lean_Elab_Command_elabNamespace_declRange__1_ LEAN_EXPORT lean_object* l_Lean_logWarning___at_Lean_Elab_Command_elabExit___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabOpen_declRange__1___closed__6; extern lean_object* l_Lean_maxRecDepth; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabExport___spec__22(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabCheck__1___closed__3; lean_object* l_List_head_x21___rarg(lean_object*, lean_object*); static lean_object* l_Lean_resolveNamespace___at_Lean_Elab_Command_elabExport___spec__1___closed__4; +static lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabVariable___spec__2(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabSynth_declRange__1___closed__7; uint8_t lean_string_dec_eq(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabCheckCore___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_withNamespace(lean_object*); +static lean_object* l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__14___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Command_elabNamespace_declRange__1___closed__3; lean_object* l_Lean_Exception_toMessageData(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabOpen___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabEnd___lambda__1___closed__5; +static lean_object* l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__19___closed__1; LEAN_EXPORT lean_object* l_Lean_resolveUniqueNamespace___at_Lean_Elab_Command_elabOpen___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabExport_declRange__1___closed__5; LEAN_EXPORT lean_object* l_Lean_activateScoped___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_addScope___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabModuleDoc_declRange__1___closed__4; +static lean_object* l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__2; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Elab_Command_elabOmit___spec__5___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_getRefPos___at_Lean_Elab_Command_elabExport___spec__20___rarg___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_string_utf8_byte_size(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabNamespace___spec__1___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___closed__12; @@ -290,7 +311,6 @@ static lean_object* l_Lean_Elab_Command_elabNamespace___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCheckCore(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Environment_registerNamespace(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabExit__1___closed__3; -LEAN_EXPORT lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCheck___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabModuleDoc_declRange__1___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Command_elabInclude__1___closed__2; @@ -298,23 +318,23 @@ LEAN_EXPORT lean_object* l_Lean_activateScoped___at___private_Lean_Elab_BuiltinC static lean_object* l___regBuiltin_Lean_Elab_Command_elabSection_declRange__1___closed__3; LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabModuleDoc___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabImport(lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__26; LEAN_EXPORT lean_object* l_Lean_Syntax_foldArgsM___at_Lean_Elab_Command_elabUniverse___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabVariable___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_mapTR_loop___at_Lean_mkConstWithLevelParams___spec__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_filterFieldList___at_Lean_Elab_Command_elabExport___spec__10___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_OpenDecl_elabOpenDecl___spec__6(size_t, size_t, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabCheckFailure_declRange__1___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Command_elabNonComputableSection__1___closed__1; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___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_Elab_Command_elabEoi(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_resolveGlobalConstNoOverloadCore___at_Lean_Elab_Command_elabExport___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__3(lean_object*, lean_object*, size_t, size_t); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8(uint8_t, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_resolveGlobalName___at_Lean_Elab_Command_elabExport___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabEnd___lambda__1___closed__8; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__12___closed__3; static lean_object* l_Lean_Elab_Command_elabEnd___lambda__1___closed__10; LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_containsId(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_popScopes___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__6; static lean_object* l___regBuiltin_Lean_Elab_Command_elabSetOption_declRange__1___closed__3; lean_object* l_Lean_InternalExceptionId_getName(lean_object*, lean_object*); static lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabNamespace___spec__1___rarg___closed__2; @@ -322,36 +342,39 @@ extern lean_object* l___private_Lean_DocString_Extension_0__Lean_moduleDocExt; LEAN_EXPORT lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_addScope___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabNonComputableSection_declRange__1___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabCheck_declRange__1(lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__20; lean_object* l_Lean_MessageData_signature(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabSetOption_declRange__1___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Command_elabAddDeclDoc__1___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Command_elabSynth__1___closed__1; lean_object* l_List_appendTR___rarg(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabEoi_declRange__1___closed__3; -static lean_object* l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabNamespace___spec__1___rarg(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Command_elabImport_declRange__1___closed__6; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOpen___spec__21___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_Command_elabOmit___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabModuleDoc__1___closed__4; size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInclude___lambda__1(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_getRefPos___at_Lean_Elab_Command_elabExport___spec__20___boxed(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabInitQuot_declRange__1___closed__2; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__12___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabExport_declRange__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabEoi___rarg(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabInitQuot__1___closed__5; static lean_object* l___regBuiltin_Lean_Elab_Command_elabNonComputableSection__1___closed__3; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabExport___spec__27(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___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__3(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabVariable_declRange__1___closed__7; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabExport___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabImport__1___closed__5; static lean_object* l___regBuiltin_Lean_Elab_Command_elabModuleDoc_declRange__1___closed__7; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_containsId___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_mapTR_loop___at_Lean_filterFieldList___spec__2(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_resolveNamespace___at_Lean_Elab_Command_elabExport___spec__1___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Command_elabSynth_declRange__1___closed__4; -LEAN_EXPORT lean_object* l_Lean_Elab_OpenDecl_resolveNameUsingNamespaces___at_Lean_Elab_Command_elabExport___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabOpen___spec__7___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabEnd_declRange__1___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Command_elabAddDeclDoc_declRange__1___closed__5; @@ -360,37 +383,37 @@ static lean_object* l___regBuiltin_Lean_Elab_Command_elabCheckFailure_declRange_ static lean_object* l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___closed__9; lean_object* l_Array_reverse___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabOpen___spec__2___rarg(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Command_elabModuleDoc___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabImport__1(lean_object*); static lean_object* l_Lean_resolveNamespace___at_Lean_Elab_Command_elabExport___spec__1___closed__1; static lean_object* l_Lean_Elab_Command_elabSection___closed__3; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Command_elabCheckCore___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_resolveGlobalConstNoOverloadCore___at_Lean_Elab_Command_elabExport___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabSection_declRange__1___closed__4; lean_object* lean_st_ref_take(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_failIfSucceeds___lambda__1___closed__2; +LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAddDeclDoc___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInitQuot___rarg___boxed(lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Elab_Command_commandElabAttribute; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabEoi_declRange__1(lean_object*); static lean_object* l_Lean_Elab_Command_elabAddDeclDoc___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSetOption___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_checkAnonymousScope(lean_object*); -LEAN_EXPORT uint8_t l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___lambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__9(uint8_t, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Command_getBracketedBinderIds(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabSetOption__1___closed__5; static lean_object* l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___closed__8; -LEAN_EXPORT uint8_t l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___lambda__2(lean_object*); lean_object* l_Lean_ResolveName_resolveNamespace(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_zip___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabSection___closed__2; static lean_object* l_Lean_Elab_Command_elabOmit___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Command_elabExit__1___closed__2; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInclude___spec__1(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_addDocString___at_Lean_Elab_Command_elabAddDeclDoc___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabSetOption_declRange__1___closed__6; static lean_object* l_Lean_Elab_Command_elabNamespace___closed__1; static lean_object* l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___closed__13; static lean_object* l___regBuiltin_Lean_Elab_Command_elabChoice_declRange__1___closed__5; static lean_object* l___regBuiltin_Lean_Elab_Command_elabInitQuot__1___closed__4; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabExport___spec__23___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint64_t lean_uint64_shift_right(uint64_t, uint64_t); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabOpen___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_SourceInfo_fromRef(lean_object*, uint8_t); @@ -401,14 +424,14 @@ LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at_Lean_Elab_Command_elabOm static lean_object* l___regBuiltin_Lean_Elab_Command_elabModuleDoc__1___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Command_elabEoi__1___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Command_elabEoi_declRange__1___closed__7; +LEAN_EXPORT lean_object* l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_div(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabEnd___lambda__1___closed__4; -static lean_object* l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__18___closed__1; +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__9; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabVariable___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabEnd_declRange__1___closed__5; lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Command_0__Lean_Elab_Command_mkTermContext___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabOmit___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*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__6; static lean_object* l___regBuiltin_Lean_Elab_Command_elabReduce_declRange__1___closed__1; lean_object* l_Lean_ScopedEnvExtension_popScope___rarg(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabModuleDoc__1___closed__8; @@ -417,36 +440,42 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandInCmd(lean_object*, lean_obje lean_object* l_Lean_Elab_Term_withoutErrToSorryImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSection(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabNonComputableSection_declRange__1___closed__4; +LEAN_EXPORT lean_object* l_Lean_Elab_addConstInfo___at_Lean_Elab_Command_elabExport___spec__23___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabNamespace_declRange__1___closed__6; uint64_t l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(lean_object*); lean_object* l_Lean_PersistentEnvExtension_addEntry___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabVersion___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_typelessBinder_x3f___closed__5; -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_getRefPos___at_Lean_Elab_Command_elabExport___spec__20___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___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___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__3; static lean_object* l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Command_elabReduce__1___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Command_elabNonComputableSection__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCheckCore___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_mkConstWithLevelParams___at_Lean_Elab_Command_elabExport___spec__24(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabModuleDoc___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Command_elabExit_declRange__1___closed__3; +LEAN_EXPORT lean_object* l_Lean_resolveGlobalName___at_Lean_Elab_Command_elabExport___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabOpen___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Command_getRef(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInitQuot(lean_object*); static lean_object* l_Lean_resolveUniqueNamespace___at_Lean_Elab_Command_elabOpen___spec__3___closed__1; static lean_object* l_Lean_Elab_Command_elabExport___closed__1; +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__38; static lean_object* l_Lean_Elab_Command_elabNonComputableSection___closed__1; +extern lean_object* l_Lean_versionString; static lean_object* l___regBuiltin_Lean_Elab_Command_elabExport__1___closed__3; lean_object* l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabExport___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__18(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabNamespace__1___closed__2; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__13___closed__1; lean_object* l_Lean_MessageData_ofFormat(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___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_Elab_getBetterRef(lean_object*, lean_object*); lean_object* l_Lean_Meta_check(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8(uint8_t, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__12___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_addScope___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabOpen_declRange__1___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Command_elabModuleDoc__1___closed__9; static lean_object* l___regBuiltin_Lean_Elab_Command_elabCheck_declRange__1___closed__1; @@ -455,20 +484,20 @@ LEAN_EXPORT lean_object* l_Lean_resolveNamespace___at_Lean_Elab_Command_elabExpo static lean_object* l___regBuiltin_Lean_Elab_Command_elabOmit__1___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabAddDeclDoc__1(lean_object*); lean_object* l_Lean_FVarId_getDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Command_elabExport___spec__17___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__28; lean_object* l_outOfBounds___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_findDeclarationRangesCore_x3f___at_Lean_Elab_Command_elabAddDeclDoc___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabAddDeclDoc___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__2(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_Command_elabOmit___spec__12(size_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_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabNamespace__1___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Command_elabEnd__1___closed__3; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandInCmd_declRange__1___closed__6; static lean_object* l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___lambda__2___closed__1; -static lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___lambda__1___closed__2; -lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__16(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__6___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Command_elabExport__1___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Command_elabVariable_declRange__1___closed__3; +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__29; lean_object* lean_st_ref_get(lean_object*, lean_object*); lean_object* l_Lean_Exception_getRef(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSynth___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -485,18 +514,20 @@ LEAN_EXPORT lean_object* l_Lean_resolveNamespace___at_Lean_Elab_Command_elabOpen LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInclude___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___regBuiltin_Lean_Elab_Command_elabCheckFailure_declRange__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabExit(lean_object*); +static lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___closed__4; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInclude___spec__1___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Command_elabSetOption__1___closed__3; lean_object* l_Lean_Syntax_getOptional_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_activateScoped___at_Lean_Elab_Command_elabOpen___spec__18___boxed(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_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___closed__4; +LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_Command_elabExport___spec__15(lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabReduce_declRange__1___closed__7; +LEAN_EXPORT lean_object* l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__14(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_to_list(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_addScopes___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__33; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInclude___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__27; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabUniverse_declRange__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabEnd___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabEnd__1___closed__1; @@ -508,10 +539,10 @@ lean_object* l_Lean_throwError___at_Lean_Elab_Term_addAutoBoundImplicits_go___sp lean_object* l_Lean_Name_append(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabOmit___lambda__2(lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabCheckFailure_declRange__1___closed__5; -LEAN_EXPORT lean_object* l_Lean_resolveGlobalName___at_Lean_Elab_Command_elabExport___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabModuleDoc_declRange__1___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabNamespace(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabExport___spec__23___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__31; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOpen___spec__17___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___closed__1; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabOpen___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -522,10 +553,9 @@ static lean_object* l___regBuiltin_Lean_Elab_Command_elabChoice__1___closed__4; static lean_object* l_Lean_resolveUniqueNamespace___at_Lean_Elab_Command_elabOpen___spec__3___closed__2; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabOpen___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Command_modifyScope(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__8; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCheckCore___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_realizeGlobalConstNoOverloadWithInfo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_ResolveName_0__Lean_resolveGlobalConstCore___at_Lean_Elab_Command_elabExport___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_addNamespace(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabSynth_declRange__1___closed__1; static lean_object* l_Lean_Elab_Command_elabModuleDoc___closed__2; @@ -535,9 +565,11 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_hasNoErrorMessages___boxed(lean_obj static lean_object* l___regBuiltin_Lean_Elab_Command_elabNamespace_declRange__1___closed__5; static lean_object* l___regBuiltin_Lean_Elab_Command_elabExport_declRange__1___closed__1; LEAN_EXPORT lean_object* l_Lean_logWarning___at_Lean_Elab_Command_elabExit___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__15(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_List_foldl___at_String_join___spec__1(lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___lambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabExit_declRange__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabEoi___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__19(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_lengthTRAux___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOpen___spec__19___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_elabAddDeclDoc(lean_object*, lean_object*, lean_object*, lean_object*); @@ -545,20 +577,20 @@ static lean_object* l___regBuiltin_Lean_Elab_Command_elabVariable_declRange__1__ static lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_addScopes___closed__1; lean_object* l_Lean_addMacroScope(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___closed__5; -static lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__11___closed__3; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabInclude__1(lean_object*); LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Elab_Command_elabOmit___spec__5(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabVariable___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabNonComputableSection_declRange__1___closed__7; -LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAddDeclDoc___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Command_elabExport___spec__18(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabNamespace_declRange__1___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Command_elabImport_declRange__1___closed__4; -LEAN_EXPORT lean_object* l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabExport___closed__4; static lean_object* l_Lean_Elab_Command_elabEnd___lambda__1___closed__2; +static lean_object* l_Lean_addDocString___at_Lean_Elab_Command_elabAddDeclDoc___spec__5___lambda__1___closed__1; uint8_t lean_name_eq(lean_object*, lean_object*); lean_object* l_List_filterMapTR_go___at_Lean_resolveNamespace___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabNamespace___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_filterFieldList___at_Lean_Elab_Command_elabExport___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabImport_declRange__1(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabUniverse_declRange__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabModuleDoc___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -566,31 +598,40 @@ static lean_object* l___regBuiltin_Lean_Elab_Command_elabEoi__1___closed__5; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabSetOption_declRange__1___closed__5; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabInitQuot__1(lean_object*); +LEAN_EXPORT lean_object* l_Lean_filterFieldList___at_Lean_Elab_Command_elabExport___spec__11___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabCheck_declRange__1___closed__6; lean_object* l_Lean_MapDeclarationExtension_find_x3f___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___lambda__2(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__16(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabAddDeclDoc_declRange__1(lean_object*); static lean_object* l_Lean_Elab_Command_elabSection___closed__4; extern lean_object* l_Lean_Elab_macroAttribute; +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_warningAsError; lean_object* l_Lean_Syntax_node2(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_mkConstWithLevelParams___at_Lean_Elab_Command_elabExport___spec__24___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabExport__1___closed__1; uint8_t l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(lean_object*, lean_object*); +extern lean_object* l_Lean_docStringExt; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabExport___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabSection_declRange__1___closed__6; static lean_object* l___regBuiltin_Lean_Elab_Command_elabEnd_declRange__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabReduce___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__36; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Elab_Command_elabOmit___spec__10(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___lambda__1___boxed(lean_object*, lean_object*, 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_addDocString___at_Lean_Elab_Command_elabAddDeclDoc___spec__5___closed__1; lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabOpen___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__26(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabChoice_declRange__1___closed__7; uint8_t l_Lean_Syntax_matchesNull(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_pushScope___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_addScope___spec__1___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabSection_declRange__1___closed__7; static lean_object* l___regBuiltin_Lean_Elab_Command_elabEoi_declRange__1___closed__5; -static lean_object* l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__3; +extern uint8_t l_System_Platform_isEmscripten; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___lambda__1(lean_object*, uint8_t, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_isIdent(lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Command_elabOpen___spec__22(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabEnd___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -598,36 +639,45 @@ extern lean_object* l_Lean_scopedEnvExtensionsRef; static lean_object* l_Lean_Elab_Command_elabEnd___lambda__1___closed__12; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInclude___spec__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAddDeclDoc___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabImport___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterTR_loop___at_Lean_Elab_Command_elabOmit___spec__15(lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabEnd__1___closed__4; +LEAN_EXPORT lean_object* l_Lean_Elab_OpenDecl_resolveId___at_Lean_Elab_Command_elabExport___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabChoice_declRange__1___closed__2; lean_object* l_Lean_Elab_Command_getScope___rarg(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandInCmd__1___closed__2; +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__35; lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_withSynthesizeImp___rarg(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Elab_Command_elabOmit___spec__6(lean_object*); lean_object* l_Lean_logAt___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_forArgsM___at_Lean_Elab_Command_elabUniverse___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabUniverse(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__5; lean_object* l_Array_eraseIdx___rarg(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__22; static lean_object* l_Lean_Elab_Command_elabImport___rarg___closed__2; +static lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__12___closed__3; LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabSynth_declRange__1___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_addConstInfo___at_Lean_Elab_Command_elabOpen___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAddDeclDoc___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_realizeGlobalConstWithInfos(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_KVMap_setBool(lean_object*, lean_object*, uint8_t); +LEAN_EXPORT lean_object* l_Lean_Elab_addConstInfo___at_Lean_Elab_Command_elabExport___spec__23(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabVariable___spec__4(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_add_alias(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__12; lean_object* l_Lean_Environment_addDecl(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInclude___spec__1___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Command_elabSynth__1___closed__5; -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabCheck__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabReduce(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Command_elabEnd_declRange__1___closed__3; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabVariable_declRange__1___closed__1; +static lean_object* l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabImport___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandInCmd___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabOpen(lean_object*, lean_object*, lean_object*, lean_object*); @@ -636,13 +686,12 @@ static lean_object* l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_elabOpen___s LEAN_EXPORT lean_object* l_Lean_popScope___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_popScopes___spec__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabCheckCore___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__11___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__32; static lean_object* l___regBuiltin_Lean_Elab_Command_elabExit_declRange__1___closed__2; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabExport___spec__21___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_resolveGlobalName___at_Lean_Elab_Command_elabExport___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_typelessBinder_x3f(lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); -lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageLog_errorsToWarnings(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Command_elabModuleDoc___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Environment_contains(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabVariable__1(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation(lean_object*, lean_object*, lean_object*, lean_object*); @@ -650,22 +699,24 @@ static lean_object* l_List_forIn_loop___at_Lean_Elab_Command_elabCheckCore___spe lean_object* l_Lean_MessageData_ofExpr(lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_expandInCmd_declRange__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_pushScope___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_addScope___spec__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Command_elabExport___spec__18___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabCheckCore___lambda__4___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___at_Lean_Elab_Command_elabAddDeclDoc___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabExit___rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__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_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___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___regBuiltin_Lean_Elab_Command_elabExit_declRange__1___closed__6; +LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAddDeclDoc___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabImport__1___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Command_elabVariable_declRange__1___closed__4; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabExport___spec__28(lean_object*, size_t, size_t, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabCheck_declRange__1___closed__5; static lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabNamespace___spec__1___rarg___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Command_elabChoice_declRange__1___closed__4; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__5; lean_object* l_Lean_Elab_Term_withAutoBoundImplicit___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterTR_loop___at_Lean_Elab_Command_elabInclude___spec__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabOmit___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabSection_declRange__1___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Command_elabAddDeclDoc_declRange__1___closed__1; -LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Command_elabExport___spec__17(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_elabChoiceAux___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabSection___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_hasNoErrorMessages___rarg___boxed(lean_object*, lean_object*); @@ -680,26 +731,30 @@ static lean_object* l___regBuiltin_Lean_Elab_Command_elabImport__1___closed__2; static lean_object* l_Lean_Elab_Command_elabOmit___lambda__1___closed__3; static lean_object* l_Lean_Elab_Command_elabAddDeclDoc___closed__2; static lean_object* l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___closed__11; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__3; -static lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___closed__2; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Elab_Command_elabOmit___spec__9(lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabUniverse__1___closed__2; static lean_object* l_Lean_Elab_Command_elabEnd___lambda__1___closed__6; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOpen___spec__17___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_typelessBinder_x3f___closed__1; lean_object* l_Lean_Elab_Command_withFreshMacroScope___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_OpenDecl_resolveNameUsingNamespaces___at_Lean_Elab_Command_elabExport___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_withNamespace___rarg(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__8___closed__1; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Elab_Command_elabOmit___spec__7(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInitQuot___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabSection_declRange__1(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabModuleDoc__1___closed__7; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabChoice_declRange__1___closed__6; lean_object* l_Lean_FileMap_leanPosToLspPos(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__7; static lean_object* l_Lean_Elab_Command_elabCheckFailure___closed__1; static lean_object* l_Lean_Elab_Command_elabCheckCore___closed__2; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOpen___spec__17___lambda__1___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Command_expandInCmd_declRange__1___closed__5; +static lean_object* l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Command_elabEoi__1___closed__4; +static lean_object* l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__4; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_resolveNamespace___at_Lean_Elab_Command_elabExport___spec__1___closed__3; lean_object* l_Lean_Elab_elabSetOption___at_Lean_withSetOptionIn___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -708,6 +763,7 @@ static lean_object* l___regBuiltin_Lean_Elab_Command_elabExport_declRange__1___c lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_OpenDecl_elabOpenDecl___spec__53(size_t, size_t, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabSynth__1___closed__3; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabUniverse__1(lean_object*); +static lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Command_elabSection__1___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Command_elabSynth_declRange__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabImport___boxed(lean_object*); @@ -720,41 +776,43 @@ static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___s static lean_object* l___regBuiltin_Lean_Elab_Command_elabSynth_declRange__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCheckCore___lambda__4(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabSynth__1___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabVersion__1(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabInitQuot_declRange__1___closed__5; extern lean_object* l_Lean_NameSet_empty; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__12___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_addScope___spec__4(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabOmit___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__21; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabEnd___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabVariable(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabImport_declRange__1___closed__5; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOpen___spec__20___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Command_elabSetOption__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_resolveGlobalConstNoOverloadCore___at_Lean_Elab_Command_elabExport___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getOptionalIdent_x3f(lean_object*); +static lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__12___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_checkEndHeader(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabExport___spec__23___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_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Command_elabInitQuot__1___closed__3; uint8_t lean_nat_dec_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabOmit___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_Command_elabExit__1(lean_object*); static lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_typelessBinder_x3f___closed__3; lean_object* l_List_drop___rarg(lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4(lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabOmit___spec__1___rarg(lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Elab_Command_elabCheckCore___spec__1___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Command_elabAddDeclDoc_declRange__1___closed__6; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___lambda__3(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_Array_mapMUnsafe_map___at_Lean_Elab_OpenDecl_elabOpenDecl___spec__5(size_t, size_t, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabSection_declRange__1___closed__2; LEAN_EXPORT lean_object* l_Lean_getConstInfo___at_Lean_Elab_Command_elabOpen___spec__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__3; static lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_typelessBinder_x3f___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSynth___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabChoice_declRange__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Command_failIfSucceeds(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__1; static lean_object* l___regBuiltin_Lean_Elab_Command_elabUniverse_declRange__1___closed__4; lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabEoi__1(lean_object*); @@ -762,13 +820,13 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Comma static lean_object* l___regBuiltin_Lean_Elab_Command_expandInCmd__1___closed__1; 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___regBuiltin_Lean_Elab_Command_elabEoi_declRange__1___closed__1; -LEAN_EXPORT lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabOpen___spec__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabReduce_go___lambda__2(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabOpen___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__13(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___regBuiltin_Lean_Elab_Command_expandInCmd_declRange__1___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Command_elabModuleDoc__1___closed__5; +LEAN_EXPORT lean_object* l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___lambda__2___boxed(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabVariable_declRange__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_failIfSucceeds___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -777,12 +835,11 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabOmit_ static lean_object* l___regBuiltin_Lean_Elab_Command_elabCheck_declRange__1___closed__7; 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___regBuiltin_Lean_Elab_Command_elabEnd_declRange__1___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_OpenDecl_resolveNameUsingNamespaces___at_Lean_Elab_Command_elabExport___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_resolveUniqueNamespace___at_Lean_Elab_Command_elabOpen___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_addConstInfo___at_Lean_Elab_Command_elabExport___spec__22(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabReduce_declRange__1___closed__6; lean_object* l_Lean_Syntax_node1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOpen___spec__20(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabModuleDoc___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Elab_Command_elabCheckCore___spec__1___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Command_elabSetOption_declRange__1___closed__1; @@ -791,37 +848,36 @@ lean_object* lean_array_set(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_addOpenDecl___at_Lean_Elab_Command_elabOpen___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_elabOpen___spec__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabInitQuot__1___closed__2; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___closed__1; -LEAN_EXPORT lean_object* l_Lean_resolveGlobalConstNoOverloadCore___at_Lean_Elab_Command_elabExport___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabModuleDoc__1___closed__10; LEAN_EXPORT lean_object* l_Lean_findDeclarationRangesCore_x3f___at_Lean_Elab_Command_elabAddDeclDoc___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabAddDeclDoc__1___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_addNamespace___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4(uint8_t, lean_object*, uint8_t, 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_elabExport___spec__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabUniverse___spec__3___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_reduce(lean_object*, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_type(lean_object*); uint64_t lean_uint64_xor(uint64_t, uint64_t); static lean_object* l___regBuiltin_Lean_Elab_Command_elabImport__1___closed__3; +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___closed__4; static lean_object* l_Lean_Elab_Command_elabEnd___lambda__1___closed__11; +static lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___lambda__1___closed__1; uint8_t l_Lean_Syntax_isNone(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabOpen___spec__2___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___lambda__1(lean_object*, uint8_t, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__2; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__3___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_elabSetOption_declRange__1___closed__7; static lean_object* l_Lean_Elab_Command_elabAddDeclDoc___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAddDeclDoc___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabExport_declRange__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCheckCore___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_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___closed__2; static lean_object* l_Lean_Elab_Command_elabModuleDoc___closed__5; -LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___at_Lean_Elab_Command_elabAddDeclDoc___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabExport___spec__27___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabVariable__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSynth___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_ResolveName_resolveGlobalName(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__18___closed__2; static lean_object* l_Lean_Elab_Command_elabVariable___closed__1; lean_object* l_Lean_Elab_Term_elabTermAndSynthesize(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_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___closed__2; @@ -829,40 +885,45 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabVa lean_object* l_Lean_Elab_Command_liftCoreM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabChoice__1(lean_object*); lean_object* lean_nat_mul(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_Command_elabExport___spec__14(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__4; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___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___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Core_resetMessageLog(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabReduce_go___lambda__2___closed__2; +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__23; static lean_object* l___regBuiltin_Lean_Elab_Command_elabNonComputableSection_declRange__1___closed__5; static lean_object* l___regBuiltin_Lean_Elab_Command_elabOpen__1___closed__3; LEAN_EXPORT lean_object* l_Lean_setEnv___at_Lean_Elab_Command_elabInitQuot___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabNonComputableSection___closed__2; +lean_object* l_Lean_Syntax_getRange_x3f(lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabOmit___spec__4___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_filterFieldList___at_Lean_Elab_Command_elabExport___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabOpen_declRange__1(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabSynth_declRange__1___closed__6; +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__26___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Command_elabModuleDoc___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_addDocString___at_Lean_Elab_Command_elabAddDeclDoc___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabEoi_declRange__1___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Command_elabExit_declRange__1___closed__7; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabExport___spec__22___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabSection__1(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabVariable__1___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabCheckFailure_declRange__1(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_toMessageList(lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Command_elabOpen___spec__22___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabVariable___spec__4___lambda__1___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3(lean_object*, uint8_t, 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__2; static lean_object* l___regBuiltin_Lean_Elab_Command_elabInitQuot_declRange__1___closed__7; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___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_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___lambda__2___closed__2; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7(uint8_t, 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_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_failIfSucceeds___closed__1; lean_object* l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___at_Lean_Elab_Command_elabAddDeclDoc___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAddDeclDoc___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Environment_getModuleIdxFor_x3f(lean_object*, lean_object*); extern lean_object* l_Lean_instInhabitedDeclarationRanges; -lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__18(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabUniverse___spec__3(lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_popScopes___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__1; lean_object* l_List_toString___at_Lean_ensureNoOverload___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Lean_activateScoped___at_Lean_Elab_Command_elabOpen___spec__18(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_reverse___rarg(lean_object*); @@ -872,16 +933,15 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabModuleDoc(lean_object*, lean_ob static lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_addScopes___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoTree___at_Lean_Elab_Command_elabOpen___spec__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCheckFailure(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___closed__1; static lean_object* l_Lean_Elab_Command_elabAddDeclDoc___closed__6; static lean_object* l_Lean_Elab_Command_elabInclude___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_OpenDecl_resolveId___at_Lean_Elab_Command_elabExport___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabCheckCore___lambda__1___closed__1; static lean_object* l_Lean_Elab_Command_elabEnd___closed__1; size_t lean_usize_sub(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_resolveNamespace___at_Lean_Elab_Command_elabOpen___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Elab_Command_instInhabitedScope; lean_object* lean_array_mk(lean_object*); -static lean_object* l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Command_elabOpen_declRange__1___closed__7; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabUniverse___closed__1; @@ -895,14 +955,17 @@ static lean_object* l_Lean_Elab_Command_elabEnd___lambda__1___closed__1; static lean_object* l_Lean_Elab_Command_elabExit___rarg___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Command_expandInCmd_declRange__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabExit___rarg___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__6; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___closed__3; lean_object* l_Lean_MessageLog_append(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getDocStringText___at_Lean_Elab_Command_elabAddDeclDoc___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandInCmd_declRange__1___closed__7; extern lean_object* l_Lean_instInhabitedName; LEAN_EXPORT lean_object* l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___at_Lean_Elab_Command_elabAddDeclDoc___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_forArgsM___at_Lean_Elab_Command_elabUniverse___spec__1___lambda__1___boxed(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_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabModuleDoc___closed__4; size_t lean_array_size(lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Command_elabOpen___spec__24(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -912,6 +975,7 @@ static lean_object* l_Lean_Elab_Command_elabModuleDoc___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Command_elabUniverse_declRange__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabReduce_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*); static lean_object* l_Lean_Elab_Command_elabAddDeclDoc___closed__1; +lean_object* l_Lean_Elab_pushInfoLeaf___at_Lean_withSetOptionIn___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_io_error_to_string(lean_object*); static lean_object* l_Lean_Elab_Command_elabSynth___lambda__2___closed__2; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabUniverse___spec__3___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -920,23 +984,27 @@ static lean_object* l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_ela static lean_object* l___regBuiltin_Lean_Elab_Command_elabImport_declRange__1___closed__2; static lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___closed__1; static lean_object* l_Lean_Elab_Command_elabCheckCore___lambda__4___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Command_elabModuleDoc___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_getRefPos___at_Lean_Elab_Command_elabExport___spec__21(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_addOpenDecl___at_Lean_Elab_Command_elabOpen___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_OpenDecl_resolveNameUsingNamespaces___at_Lean_Elab_Command_elabExport___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__3; +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__25; static lean_object* l___regBuiltin_Lean_Elab_Command_elabOpen__1___closed__1; -LEAN_EXPORT lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static uint8_t l_Lean_Elab_Command_elabVersion___rarg___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_elabOpen___spec__15(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___closed__6; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabOpen__1(lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___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_string_append(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabExport___spec__27___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__11(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabReduce_declRange__1(lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__37; static lean_object* l___regBuiltin_Lean_Elab_Command_elabEoi_declRange__1___closed__6; static lean_object* l___regBuiltin_Lean_Elab_Command_elabUniverse__1___closed__4; -LEAN_EXPORT lean_object* l_Lean_filterFieldList___at_Lean_Elab_Command_elabExport___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSynth(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabNamespace__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabOpen___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -946,24 +1014,21 @@ lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Syntax_SepArray_getElems___spec static lean_object* l___regBuiltin_Lean_Elab_Command_elabReduce_declRange__1___closed__2; lean_object* lean_array_get_size(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabEnd_declRange__1___closed__7; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_resolveNamespace___at_Lean_Elab_Command_elabExport___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_getDocStringText___at_Lean_Elab_Command_elabAddDeclDoc___spec__2___closed__1; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Command_elabAddDeclDoc_declRange__1___closed__4; -LEAN_EXPORT lean_object* l_Lean_getRefPos___at_Lean_Elab_Command_elabExport___spec__20(lean_object*); +LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_Command_elabExport___spec__17(lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabInclude__1___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Command_elabImport_declRange__1___closed__7; static lean_object* l___regBuiltin_Lean_Elab_Command_elabNamespace__1___closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__18___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutErrToSorry___at_Lean_Elab_Command_elabOmit___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabEoi_declRange__1___closed__2; -static lean_object* l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__13___closed__1; extern lean_object* l_Lean_Elab_unsupportedSyntaxExceptionId; -LEAN_EXPORT lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___closed__4; +LEAN_EXPORT lean_object* l___private_Lean_ResolveName_0__Lean_resolveGlobalConstCore___at_Lean_Elab_Command_elabExport___spec__9___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_Elab_BuiltinCommand_0__Lean_Elab_Command_elabChoiceAux(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_mkArray2___rarg(lean_object*, lean_object*); @@ -971,14 +1036,15 @@ static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCom static lean_object* l___regBuiltin_Lean_Elab_Command_elabOpen_declRange__1___closed__5; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabVariable___spec__4___lambda__1(lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabExport_declRange__1___closed__7; -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabExport___spec__24(lean_object*, size_t, size_t, lean_object*); +lean_object* l_Lean_throwError___at_Lean_withSetOptionIn___spec__7(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___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_expr_dbg_to_string(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_addScope(uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabExit_declRange__1___closed__5; static lean_object* l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___closed__10; lean_object* lean_nat_add(lean_object*, lean_object*); static lean_object* l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_elabOpen___spec__15___closed__3; -LEAN_EXPORT lean_object* l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___lambda__2___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Exception_isRuntime(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSynth___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_throwError___at_Lean_Elab_Command_elabAddDeclDoc___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); @@ -987,51 +1053,62 @@ static lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_ch lean_object* l_List_toString___at_Lean_OpenDecl_instToString___spec__1(lean_object*); static lean_object* l_Lean_Elab_Command_elabReduce___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSetOption(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__2; +extern lean_object* l_System_Platform_target; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabExport___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__19___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabVariable___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterTR_loop___at_Lean_Elab_Command_elabInclude___spec__2(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__40; +extern uint8_t l_System_Platform_isWindows; lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___spec__2(size_t, size_t, lean_object*); lean_object* l_Lean_KernelException_toMessageData(lean_object*, lean_object*); -lean_object* l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_expandDeclId___spec__11(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__5; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabExport___spec__27___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabCheck_declRange__1___closed__3; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabAddDeclDoc___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabNonComputableSection(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabInitQuot_declRange__1___closed__4; -LEAN_EXPORT lean_object* l___private_Lean_ResolveName_0__Lean_resolveGlobalConstCore___at_Lean_Elab_Command_elabExport___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_uset(lean_object*, size_t, lean_object*); lean_object* l_Lean_MessageData_ofName(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOpen___spec__23(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabOpen_declRange__1___closed__1; lean_object* l___private_Init_Data_Repr_0__Nat_reprFast(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabChoice__1___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Command_elabOpen__1___closed__2; +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__13; +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__41; lean_object* l_List_filterTR_loop___at_Lean_filterFieldList___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabEnd___closed__2; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCheckCore___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___regBuiltin_Lean_Elab_Command_elabOmit__1(lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___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_List_mapTR_loop___at_Lean_Elab_Command_elabExport___spec__16(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_failIfSucceeds___lambda__1___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Command_elabNonComputableSection_declRange__1___closed__1; uint8_t l_Lean_Expr_isSyntheticSorry(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabOpen___lambda__1(lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__3___closed__1; static lean_object* l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___closed__7; LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoTree___at_Lean_Elab_Command_elabOpen___spec__16(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at_Lean_Elab_Command_elabOmit___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___private_Lean_ResolveName_0__Lean_resolveGlobalConstCore___at_Lean_Elab_Command_elabExport___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_getRefPos___at_Lean_Elab_Command_elabExport___spec__21___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSetOption___lambda__1(lean_object*, lean_object*); size_t lean_usize_land(size_t, size_t); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOpen___spec__25(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabOmit__1___closed__3; LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_Command_elabEnd___spec__1(lean_object*, lean_object*); -static lean_object* l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__13___closed__2; +static lean_object* l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAddDeclDoc___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__19___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCheckCore___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 uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_containsId___spec__1(lean_object*, lean_object*, size_t, size_t); static lean_object* l___regBuiltin_Lean_Elab_Command_expandInCmd_declRange__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at_Lean_Elab_Command_elabExport___spec__25___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabOmit__1___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabNonComputableSection__1(lean_object*); +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at_Lean_Elab_Command_elabExport___spec__25(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_MessageLog_hasErrors(lean_object*); lean_object* l_Lean_Elab_Term_withDeclName___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabModuleDoc___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { @@ -1096,237 +1173,146 @@ return x_24; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Command_elabModuleDoc___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Command_elabModuleDoc___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_5; uint8_t x_6; lean_object* x_7; lean_object* x_8; -x_5 = lean_ctor_get(x_2, 1); -lean_inc(x_5); -lean_dec(x_2); -x_6 = 0; -x_7 = l_Lean_Syntax_getPos_x3f(x_1, x_6); -x_8 = l_Lean_Syntax_getTailPos_x3f(x_1, x_6); -if (lean_obj_tag(x_7) == 0) +uint8_t x_5; lean_object* x_6; +x_5 = 0; +x_6 = l_Lean_Syntax_getRange_x3f(x_1, x_5); +if (lean_obj_tag(x_6) == 0) { -lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_9 = lean_unsigned_to_nat(0u); -lean_inc(x_5); -x_10 = l_Lean_FileMap_toPosition(x_5, x_9); -lean_inc(x_10); -x_11 = l_Lean_FileMap_leanPosToLspPos(x_5, x_10); -if (lean_obj_tag(x_8) == 0) +lean_object* x_7; lean_object* x_8; +lean_dec(x_2); +x_7 = lean_box(0); +x_8 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_8, 0, x_7); +lean_ctor_set(x_8, 1, x_4); +return x_8; +} +else { -uint8_t x_12; -lean_dec(x_5); -x_12 = !lean_is_exclusive(x_11); -if (x_12 == 0) +uint8_t x_9; +x_9 = !lean_is_exclusive(x_6); +if (x_9 == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_ctor_get(x_11, 1); -x_14 = lean_ctor_get(x_11, 0); +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_10 = lean_ctor_get(x_6, 0); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); +lean_dec(x_2); +x_12 = lean_ctor_get(x_10, 0); +lean_inc(x_12); +lean_inc(x_11); +x_13 = l_Lean_FileMap_toPosition(x_11, x_12); +lean_dec(x_12); +x_14 = lean_ctor_get(x_10, 1); +lean_inc(x_14); +lean_dec(x_10); +lean_inc(x_11); +x_15 = l_Lean_FileMap_toPosition(x_11, x_14); lean_dec(x_14); lean_inc(x_13); -lean_inc(x_10); -x_15 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_15, 0, x_10); -lean_ctor_set(x_15, 1, x_13); -lean_ctor_set(x_15, 2, x_10); -lean_ctor_set(x_15, 3, x_13); -lean_ctor_set(x_11, 1, x_4); -lean_ctor_set(x_11, 0, x_15); -return x_11; -} -else +x_16 = l_Lean_FileMap_leanPosToLspPos(x_11, x_13); +x_17 = !lean_is_exclusive(x_16); +if (x_17 == 0) { -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_11, 1); -lean_inc(x_16); +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_18 = lean_ctor_get(x_16, 1); +x_19 = lean_ctor_get(x_16, 0); +lean_dec(x_19); +lean_inc(x_15); +x_20 = l_Lean_FileMap_leanPosToLspPos(x_11, x_15); lean_dec(x_11); -lean_inc(x_16); -lean_inc(x_10); -x_17 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_17, 0, x_10); -lean_ctor_set(x_17, 1, x_16); -lean_ctor_set(x_17, 2, x_10); -lean_ctor_set(x_17, 3, x_16); -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_17); -lean_ctor_set(x_18, 1, x_4); -return x_18; -} +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +x_22 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_22, 0, x_13); +lean_ctor_set(x_22, 1, x_18); +lean_ctor_set(x_22, 2, x_15); +lean_ctor_set(x_22, 3, x_21); +lean_ctor_set(x_6, 0, x_22); +lean_ctor_set(x_16, 1, x_4); +lean_ctor_set(x_16, 0, x_6); +return x_16; } else { -uint8_t x_19; -x_19 = !lean_is_exclusive(x_11); -if (x_19 == 0) -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_20 = lean_ctor_get(x_11, 1); -x_21 = lean_ctor_get(x_11, 0); -lean_dec(x_21); -x_22 = lean_ctor_get(x_8, 0); -lean_inc(x_22); -lean_dec(x_8); -lean_inc(x_5); -x_23 = l_Lean_FileMap_toPosition(x_5, x_22); -lean_dec(x_22); +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_23 = lean_ctor_get(x_16, 1); lean_inc(x_23); -x_24 = l_Lean_FileMap_leanPosToLspPos(x_5, x_23); -lean_dec(x_5); +lean_dec(x_16); +lean_inc(x_15); +x_24 = l_Lean_FileMap_leanPosToLspPos(x_11, x_15); +lean_dec(x_11); x_25 = lean_ctor_get(x_24, 1); lean_inc(x_25); lean_dec(x_24); x_26 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_26, 0, x_10); -lean_ctor_set(x_26, 1, x_20); -lean_ctor_set(x_26, 2, x_23); +lean_ctor_set(x_26, 0, x_13); +lean_ctor_set(x_26, 1, x_23); +lean_ctor_set(x_26, 2, x_15); lean_ctor_set(x_26, 3, x_25); -lean_ctor_set(x_11, 1, x_4); -lean_ctor_set(x_11, 0, x_26); -return x_11; +lean_ctor_set(x_6, 0, x_26); +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_6); +lean_ctor_set(x_27, 1, x_4); +return x_27; +} } else { -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_27 = lean_ctor_get(x_11, 1); -lean_inc(x_27); -lean_dec(x_11); -x_28 = lean_ctor_get(x_8, 0); +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_28 = lean_ctor_get(x_6, 0); lean_inc(x_28); -lean_dec(x_8); -lean_inc(x_5); -x_29 = l_Lean_FileMap_toPosition(x_5, x_28); +lean_dec(x_6); +x_29 = lean_ctor_get(x_2, 1); +lean_inc(x_29); +lean_dec(x_2); +x_30 = lean_ctor_get(x_28, 0); +lean_inc(x_30); +lean_inc(x_29); +x_31 = l_Lean_FileMap_toPosition(x_29, x_30); +lean_dec(x_30); +x_32 = lean_ctor_get(x_28, 1); +lean_inc(x_32); lean_dec(x_28); lean_inc(x_29); -x_30 = l_Lean_FileMap_leanPosToLspPos(x_5, x_29); -lean_dec(x_5); -x_31 = lean_ctor_get(x_30, 1); +x_33 = l_Lean_FileMap_toPosition(x_29, x_32); +lean_dec(x_32); lean_inc(x_31); -lean_dec(x_30); -x_32 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_32, 0, x_10); -lean_ctor_set(x_32, 1, x_27); -lean_ctor_set(x_32, 2, x_29); -lean_ctor_set(x_32, 3, x_31); -x_33 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_33, 0, x_32); -lean_ctor_set(x_33, 1, x_4); -return x_33; -} -} -} -else -{ -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_7, 0); -lean_inc(x_34); -lean_dec(x_7); -lean_inc(x_5); -x_35 = l_Lean_FileMap_toPosition(x_5, x_34); -lean_dec(x_34); -lean_inc(x_35); -x_36 = l_Lean_FileMap_leanPosToLspPos(x_5, x_35); -if (lean_obj_tag(x_8) == 0) -{ -uint8_t x_37; -lean_dec(x_5); -x_37 = !lean_is_exclusive(x_36); -if (x_37 == 0) -{ -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_36, 1); -x_39 = lean_ctor_get(x_36, 0); -lean_dec(x_39); -lean_inc(x_38); -lean_inc(x_35); -x_40 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_40, 0, x_35); -lean_ctor_set(x_40, 1, x_38); -lean_ctor_set(x_40, 2, x_35); -lean_ctor_set(x_40, 3, x_38); -lean_ctor_set(x_36, 1, x_4); -lean_ctor_set(x_36, 0, x_40); -return x_36; -} -else -{ -lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_ctor_get(x_36, 1); -lean_inc(x_41); -lean_dec(x_36); -lean_inc(x_41); +x_34 = l_Lean_FileMap_leanPosToLspPos(x_29, x_31); +x_35 = lean_ctor_get(x_34, 1); lean_inc(x_35); -x_42 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_42, 0, x_35); -lean_ctor_set(x_42, 1, x_41); -lean_ctor_set(x_42, 2, x_35); -lean_ctor_set(x_42, 3, x_41); -x_43 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_43, 0, x_42); -lean_ctor_set(x_43, 1, x_4); -return x_43; -} -} -else -{ -uint8_t x_44; -x_44 = !lean_is_exclusive(x_36); -if (x_44 == 0) -{ -lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_45 = lean_ctor_get(x_36, 1); -x_46 = lean_ctor_get(x_36, 0); -lean_dec(x_46); -x_47 = lean_ctor_get(x_8, 0); -lean_inc(x_47); -lean_dec(x_8); -lean_inc(x_5); -x_48 = l_Lean_FileMap_toPosition(x_5, x_47); -lean_dec(x_47); -lean_inc(x_48); -x_49 = l_Lean_FileMap_leanPosToLspPos(x_5, x_48); -lean_dec(x_5); -x_50 = lean_ctor_get(x_49, 1); -lean_inc(x_50); -lean_dec(x_49); -x_51 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_51, 0, x_35); -lean_ctor_set(x_51, 1, x_45); -lean_ctor_set(x_51, 2, x_48); -lean_ctor_set(x_51, 3, x_50); -lean_ctor_set(x_36, 1, x_4); -lean_ctor_set(x_36, 0, x_51); -return x_36; +if (lean_is_exclusive(x_34)) { + lean_ctor_release(x_34, 0); + lean_ctor_release(x_34, 1); + x_36 = x_34; +} else { + lean_dec_ref(x_34); + x_36 = lean_box(0); } -else -{ -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; -x_52 = lean_ctor_get(x_36, 1); -lean_inc(x_52); -lean_dec(x_36); -x_53 = lean_ctor_get(x_8, 0); -lean_inc(x_53); -lean_dec(x_8); -lean_inc(x_5); -x_54 = l_Lean_FileMap_toPosition(x_5, x_53); -lean_dec(x_53); -lean_inc(x_54); -x_55 = l_Lean_FileMap_leanPosToLspPos(x_5, x_54); -lean_dec(x_5); -x_56 = lean_ctor_get(x_55, 1); -lean_inc(x_56); -lean_dec(x_55); -x_57 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_57, 0, x_35); -lean_ctor_set(x_57, 1, x_52); -lean_ctor_set(x_57, 2, x_54); -lean_ctor_set(x_57, 3, x_56); -x_58 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_58, 0, x_57); -lean_ctor_set(x_58, 1, x_4); -return x_58; +lean_inc(x_33); +x_37 = l_Lean_FileMap_leanPosToLspPos(x_29, x_33); +lean_dec(x_29); +x_38 = lean_ctor_get(x_37, 1); +lean_inc(x_38); +lean_dec(x_37); +x_39 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_39, 0, x_31); +lean_ctor_set(x_39, 1, x_35); +lean_ctor_set(x_39, 2, x_33); +lean_ctor_set(x_39, 3, x_38); +x_40 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_40, 0, x_39); +if (lean_is_scalar(x_36)) { + x_41 = lean_alloc_ctor(0, 2, 0); +} else { + x_41 = x_36; } +lean_ctor_set(x_41, 0, x_40); +lean_ctor_set(x_41, 1, x_4); +return x_41; } } } @@ -1381,7 +1367,7 @@ x_5 = lean_unsigned_to_nat(1u); x_6 = l_Lean_Syntax_getArg(x_1, x_5); if (lean_obj_tag(x_6) == 2) { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; x_7 = lean_ctor_get(x_6, 1); lean_inc(x_7); lean_dec(x_6); @@ -1393,202 +1379,236 @@ x_11 = lean_unsigned_to_nat(0u); x_12 = lean_string_utf8_extract(x_7, x_11, x_10); lean_dec(x_10); lean_dec(x_7); -x_13 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Command_elabModuleDoc___spec__2(x_1, x_2, x_3, x_4); +x_13 = l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Command_elabModuleDoc___spec__2(x_1, x_2, x_3, x_4); x_14 = lean_ctor_get(x_13, 0); lean_inc(x_14); -x_15 = lean_ctor_get(x_13, 1); -lean_inc(x_15); +if (lean_obj_tag(x_14) == 0) +{ +uint8_t x_15; +lean_dec(x_12); +x_15 = !lean_is_exclusive(x_13); +if (x_15 == 0) +{ +lean_object* x_16; lean_object* x_17; +x_16 = lean_ctor_get(x_13, 0); +lean_dec(x_16); +x_17 = lean_box(0); +lean_ctor_set(x_13, 0, x_17); +return x_13; +} +else +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_13, 1); +lean_inc(x_18); lean_dec(x_13); -x_16 = lean_st_ref_take(x_3, x_15); -x_17 = !lean_is_exclusive(x_16); -if (x_17 == 0) +x_19 = lean_box(0); +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_19); +lean_ctor_set(x_20, 1, x_18); +return x_20; +} +} +else { -lean_object* x_18; uint8_t x_19; -x_18 = lean_ctor_get(x_16, 0); -x_19 = !lean_is_exclusive(x_18); -if (x_19 == 0) +lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; +x_21 = lean_ctor_get(x_13, 1); +lean_inc(x_21); +lean_dec(x_13); +x_22 = lean_ctor_get(x_14, 0); +lean_inc(x_22); +lean_dec(x_14); +x_23 = lean_st_ref_take(x_3, x_21); +x_24 = !lean_is_exclusive(x_23); +if (x_24 == 0) { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; -x_20 = lean_ctor_get(x_16, 1); -x_21 = lean_ctor_get(x_18, 0); -lean_ctor_set(x_16, 1, x_14); -lean_ctor_set(x_16, 0, x_12); -x_22 = l_Lean_Elab_Command_elabModuleDoc___closed__5; -x_23 = l_Lean_PersistentEnvExtension_addEntry___rarg(x_22, x_21, x_16); -lean_ctor_set(x_18, 0, x_23); -x_24 = lean_st_ref_set(x_3, x_18, x_20); -x_25 = !lean_is_exclusive(x_24); -if (x_25 == 0) +lean_object* x_25; uint8_t x_26; +x_25 = lean_ctor_get(x_23, 0); +x_26 = !lean_is_exclusive(x_25); +if (x_26 == 0) { -lean_object* x_26; lean_object* x_27; -x_26 = lean_ctor_get(x_24, 0); -lean_dec(x_26); -x_27 = lean_box(0); -lean_ctor_set(x_24, 0, x_27); -return x_24; +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; +x_27 = lean_ctor_get(x_23, 1); +x_28 = lean_ctor_get(x_25, 0); +lean_ctor_set(x_23, 1, x_22); +lean_ctor_set(x_23, 0, x_12); +x_29 = l_Lean_Elab_Command_elabModuleDoc___closed__5; +x_30 = l_Lean_PersistentEnvExtension_addEntry___rarg(x_29, x_28, x_23); +lean_ctor_set(x_25, 0, x_30); +x_31 = lean_st_ref_set(x_3, x_25, x_27); +x_32 = !lean_is_exclusive(x_31); +if (x_32 == 0) +{ +lean_object* x_33; lean_object* x_34; +x_33 = lean_ctor_get(x_31, 0); +lean_dec(x_33); +x_34 = lean_box(0); +lean_ctor_set(x_31, 0, x_34); +return x_31; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_28 = lean_ctor_get(x_24, 1); -lean_inc(x_28); -lean_dec(x_24); -x_29 = lean_box(0); -x_30 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_30, 0, x_29); -lean_ctor_set(x_30, 1, x_28); -return x_30; +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_31, 1); +lean_inc(x_35); +lean_dec(x_31); +x_36 = lean_box(0); +x_37 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_37, 0, x_36); +lean_ctor_set(x_37, 1, x_35); +return x_37; } } else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_31 = lean_ctor_get(x_16, 1); -x_32 = lean_ctor_get(x_18, 0); -x_33 = lean_ctor_get(x_18, 1); -x_34 = lean_ctor_get(x_18, 2); -x_35 = lean_ctor_get(x_18, 3); -x_36 = lean_ctor_get(x_18, 4); -x_37 = lean_ctor_get(x_18, 5); -x_38 = lean_ctor_get(x_18, 6); -x_39 = lean_ctor_get(x_18, 7); -lean_inc(x_39); -lean_inc(x_38); -lean_inc(x_37); -lean_inc(x_36); -lean_inc(x_35); -lean_inc(x_34); -lean_inc(x_33); -lean_inc(x_32); -lean_dec(x_18); -lean_ctor_set(x_16, 1, x_14); -lean_ctor_set(x_16, 0, x_12); -x_40 = l_Lean_Elab_Command_elabModuleDoc___closed__5; -x_41 = l_Lean_PersistentEnvExtension_addEntry___rarg(x_40, x_32, x_16); -x_42 = lean_alloc_ctor(0, 8, 0); -lean_ctor_set(x_42, 0, x_41); -lean_ctor_set(x_42, 1, x_33); -lean_ctor_set(x_42, 2, x_34); -lean_ctor_set(x_42, 3, x_35); -lean_ctor_set(x_42, 4, x_36); -lean_ctor_set(x_42, 5, x_37); -lean_ctor_set(x_42, 6, x_38); -lean_ctor_set(x_42, 7, x_39); -x_43 = lean_st_ref_set(x_3, x_42, x_31); -x_44 = lean_ctor_get(x_43, 1); +lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_38 = lean_ctor_get(x_23, 1); +x_39 = lean_ctor_get(x_25, 0); +x_40 = lean_ctor_get(x_25, 1); +x_41 = lean_ctor_get(x_25, 2); +x_42 = lean_ctor_get(x_25, 3); +x_43 = lean_ctor_get(x_25, 4); +x_44 = lean_ctor_get(x_25, 5); +x_45 = lean_ctor_get(x_25, 6); +x_46 = lean_ctor_get(x_25, 7); +lean_inc(x_46); +lean_inc(x_45); lean_inc(x_44); -if (lean_is_exclusive(x_43)) { - lean_ctor_release(x_43, 0); - lean_ctor_release(x_43, 1); - x_45 = x_43; +lean_inc(x_43); +lean_inc(x_42); +lean_inc(x_41); +lean_inc(x_40); +lean_inc(x_39); +lean_dec(x_25); +lean_ctor_set(x_23, 1, x_22); +lean_ctor_set(x_23, 0, x_12); +x_47 = l_Lean_Elab_Command_elabModuleDoc___closed__5; +x_48 = l_Lean_PersistentEnvExtension_addEntry___rarg(x_47, x_39, x_23); +x_49 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_49, 0, x_48); +lean_ctor_set(x_49, 1, x_40); +lean_ctor_set(x_49, 2, x_41); +lean_ctor_set(x_49, 3, x_42); +lean_ctor_set(x_49, 4, x_43); +lean_ctor_set(x_49, 5, x_44); +lean_ctor_set(x_49, 6, x_45); +lean_ctor_set(x_49, 7, x_46); +x_50 = lean_st_ref_set(x_3, x_49, x_38); +x_51 = lean_ctor_get(x_50, 1); +lean_inc(x_51); +if (lean_is_exclusive(x_50)) { + lean_ctor_release(x_50, 0); + lean_ctor_release(x_50, 1); + x_52 = x_50; } else { - lean_dec_ref(x_43); - x_45 = lean_box(0); + lean_dec_ref(x_50); + x_52 = lean_box(0); } -x_46 = lean_box(0); -if (lean_is_scalar(x_45)) { - x_47 = lean_alloc_ctor(0, 2, 0); +x_53 = lean_box(0); +if (lean_is_scalar(x_52)) { + x_54 = lean_alloc_ctor(0, 2, 0); } else { - x_47 = x_45; + x_54 = x_52; } -lean_ctor_set(x_47, 0, x_46); -lean_ctor_set(x_47, 1, x_44); -return x_47; +lean_ctor_set(x_54, 0, x_53); +lean_ctor_set(x_54, 1, x_51); +return x_54; } } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; -x_48 = lean_ctor_get(x_16, 0); -x_49 = lean_ctor_get(x_16, 1); -lean_inc(x_49); -lean_inc(x_48); -lean_dec(x_16); -x_50 = lean_ctor_get(x_48, 0); -lean_inc(x_50); -x_51 = lean_ctor_get(x_48, 1); -lean_inc(x_51); -x_52 = lean_ctor_get(x_48, 2); -lean_inc(x_52); -x_53 = lean_ctor_get(x_48, 3); -lean_inc(x_53); -x_54 = lean_ctor_get(x_48, 4); -lean_inc(x_54); -x_55 = lean_ctor_get(x_48, 5); -lean_inc(x_55); -x_56 = lean_ctor_get(x_48, 6); +lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; +x_55 = lean_ctor_get(x_23, 0); +x_56 = lean_ctor_get(x_23, 1); lean_inc(x_56); -x_57 = lean_ctor_get(x_48, 7); +lean_inc(x_55); +lean_dec(x_23); +x_57 = lean_ctor_get(x_55, 0); lean_inc(x_57); -if (lean_is_exclusive(x_48)) { - lean_ctor_release(x_48, 0); - lean_ctor_release(x_48, 1); - lean_ctor_release(x_48, 2); - lean_ctor_release(x_48, 3); - lean_ctor_release(x_48, 4); - lean_ctor_release(x_48, 5); - lean_ctor_release(x_48, 6); - lean_ctor_release(x_48, 7); - x_58 = x_48; -} else { - lean_dec_ref(x_48); - x_58 = lean_box(0); -} -x_59 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_59, 0, x_12); -lean_ctor_set(x_59, 1, x_14); -x_60 = l_Lean_Elab_Command_elabModuleDoc___closed__5; -x_61 = l_Lean_PersistentEnvExtension_addEntry___rarg(x_60, x_50, x_59); -if (lean_is_scalar(x_58)) { - x_62 = lean_alloc_ctor(0, 8, 0); -} else { - x_62 = x_58; -} -lean_ctor_set(x_62, 0, x_61); -lean_ctor_set(x_62, 1, x_51); -lean_ctor_set(x_62, 2, x_52); -lean_ctor_set(x_62, 3, x_53); -lean_ctor_set(x_62, 4, x_54); -lean_ctor_set(x_62, 5, x_55); -lean_ctor_set(x_62, 6, x_56); -lean_ctor_set(x_62, 7, x_57); -x_63 = lean_st_ref_set(x_3, x_62, x_49); -x_64 = lean_ctor_get(x_63, 1); +x_58 = lean_ctor_get(x_55, 1); +lean_inc(x_58); +x_59 = lean_ctor_get(x_55, 2); +lean_inc(x_59); +x_60 = lean_ctor_get(x_55, 3); +lean_inc(x_60); +x_61 = lean_ctor_get(x_55, 4); +lean_inc(x_61); +x_62 = lean_ctor_get(x_55, 5); +lean_inc(x_62); +x_63 = lean_ctor_get(x_55, 6); +lean_inc(x_63); +x_64 = lean_ctor_get(x_55, 7); lean_inc(x_64); -if (lean_is_exclusive(x_63)) { - lean_ctor_release(x_63, 0); - lean_ctor_release(x_63, 1); - x_65 = x_63; -} else { - lean_dec_ref(x_63); +if (lean_is_exclusive(x_55)) { + lean_ctor_release(x_55, 0); + lean_ctor_release(x_55, 1); + lean_ctor_release(x_55, 2); + lean_ctor_release(x_55, 3); + lean_ctor_release(x_55, 4); + lean_ctor_release(x_55, 5); + lean_ctor_release(x_55, 6); + lean_ctor_release(x_55, 7); + x_65 = x_55; +} else { + lean_dec_ref(x_55); x_65 = lean_box(0); } -x_66 = lean_box(0); +x_66 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_66, 0, x_12); +lean_ctor_set(x_66, 1, x_22); +x_67 = l_Lean_Elab_Command_elabModuleDoc___closed__5; +x_68 = l_Lean_PersistentEnvExtension_addEntry___rarg(x_67, x_57, x_66); if (lean_is_scalar(x_65)) { - x_67 = lean_alloc_ctor(0, 2, 0); + x_69 = lean_alloc_ctor(0, 8, 0); } else { - x_67 = x_65; + x_69 = x_65; +} +lean_ctor_set(x_69, 0, x_68); +lean_ctor_set(x_69, 1, x_58); +lean_ctor_set(x_69, 2, x_59); +lean_ctor_set(x_69, 3, x_60); +lean_ctor_set(x_69, 4, x_61); +lean_ctor_set(x_69, 5, x_62); +lean_ctor_set(x_69, 6, x_63); +lean_ctor_set(x_69, 7, x_64); +x_70 = lean_st_ref_set(x_3, x_69, x_56); +x_71 = lean_ctor_get(x_70, 1); +lean_inc(x_71); +if (lean_is_exclusive(x_70)) { + lean_ctor_release(x_70, 0); + lean_ctor_release(x_70, 1); + x_72 = x_70; +} else { + lean_dec_ref(x_70); + x_72 = lean_box(0); +} +x_73 = lean_box(0); +if (lean_is_scalar(x_72)) { + x_74 = lean_alloc_ctor(0, 2, 0); +} else { + x_74 = x_72; +} +lean_ctor_set(x_74, 0, x_73); +lean_ctor_set(x_74, 1, x_71); +return x_74; } -lean_ctor_set(x_67, 0, x_66); -lean_ctor_set(x_67, 1, x_64); -return x_67; } } else { -lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; -x_68 = l_Lean_MessageData_ofSyntax(x_6); -x_69 = l_Lean_indentD(x_68); -x_70 = l_Lean_Elab_Command_elabModuleDoc___closed__2; -x_71 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_71, 0, x_70); -lean_ctor_set(x_71, 1, x_69); -x_72 = l_Lean_Elab_Command_elabModuleDoc___closed__4; -x_73 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_73, 0, x_71); -lean_ctor_set(x_73, 1, x_72); -x_74 = l_Lean_throwErrorAt___at_Lean_Elab_Command_elabModuleDoc___spec__1(x_1, x_73, x_2, x_3, x_4); -return x_74; +lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_75 = l_Lean_MessageData_ofSyntax(x_6); +x_76 = l_Lean_indentD(x_75); +x_77 = l_Lean_Elab_Command_elabModuleDoc___closed__2; +x_78 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_78, 0, x_77); +lean_ctor_set(x_78, 1, x_76); +x_79 = l_Lean_Elab_Command_elabModuleDoc___closed__4; +x_80 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_80, 0, x_78); +lean_ctor_set(x_80, 1, x_79); +x_81 = l_Lean_throwErrorAt___at_Lean_Elab_Command_elabModuleDoc___spec__1(x_1, x_80, x_2, x_3, x_4); +return x_81; } } } @@ -1602,11 +1622,11 @@ lean_dec(x_1); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Command_elabModuleDoc___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Command_elabModuleDoc___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Command_elabModuleDoc___spec__2(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Command_elabModuleDoc___spec__2(x_1, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_1); return x_5; @@ -6072,6 +6092,94 @@ x_4 = l_Lean_addBuiltinDeclarationRanges(x_2, x_3, x_1); return x_4; } } +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_5 = l_Lean_Elab_Command_getRef(x_2, x_3, x_4); +x_6 = lean_ctor_get(x_5, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_5, 1); +lean_inc(x_7); +lean_dec(x_5); +x_8 = lean_ctor_get(x_2, 4); +lean_inc(x_8); +lean_inc(x_8); +x_9 = l_Lean_Elab_getBetterRef(x_6, x_8); +lean_dec(x_6); +x_10 = l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1(x_1, x_2, x_3, x_7); +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_12 = lean_ctor_get(x_10, 0); +x_13 = lean_ctor_get(x_10, 1); +x_14 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_12, x_8, x_2, x_3, x_13); +lean_dec(x_2); +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 0) +{ +lean_object* x_16; +x_16 = lean_ctor_get(x_14, 0); +lean_ctor_set(x_10, 1, x_16); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set_tag(x_14, 1); +lean_ctor_set(x_14, 0, x_10); +return x_14; +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_14, 0); +x_18 = lean_ctor_get(x_14, 1); +lean_inc(x_18); +lean_inc(x_17); +lean_dec(x_14); +lean_ctor_set(x_10, 1, x_17); +lean_ctor_set(x_10, 0, x_9); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_10); +lean_ctor_set(x_19, 1, 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; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_20 = lean_ctor_get(x_10, 0); +x_21 = lean_ctor_get(x_10, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_10); +x_22 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_20, x_8, x_2, x_3, x_21); +lean_dec(x_2); +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +if (lean_is_exclusive(x_22)) { + lean_ctor_release(x_22, 0); + lean_ctor_release(x_22, 1); + x_25 = x_22; +} else { + lean_dec_ref(x_22); + x_25 = lean_box(0); +} +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_9); +lean_ctor_set(x_26, 1, x_23); +if (lean_is_scalar(x_25)) { + x_27 = lean_alloc_ctor(1, 2, 0); +} else { + x_27 = x_25; + lean_ctor_set_tag(x_27, 1); +} +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_24); +return x_27; +} +} +} LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabExport___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { @@ -6091,7 +6199,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_expandDeclId___spec__16(x_2, x_3, x_4, x_8); +x_12 = l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__3(x_2, x_3, x_4, x_8); return x_12; } else @@ -6129,12 +6237,12 @@ lean_ctor_set(x_23, 7, x_19); lean_ctor_set(x_23, 8, x_20); lean_ctor_set(x_23, 9, x_21); lean_ctor_set_uint8(x_23, sizeof(void*)*10, x_22); -x_24 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__16(x_2, x_23, x_4, x_8); +x_24 = l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__3(x_2, x_23, x_4, x_8); return x_24; } } } -LEAN_EXPORT lean_object* l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___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_EXPORT lean_object* l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___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; @@ -6144,7 +6252,7 @@ lean_ctor_set(x_6, 1, x_5); return x_6; } } -LEAN_EXPORT uint8_t l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___lambda__2(lean_object* x_1) { +LEAN_EXPORT uint8_t l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___lambda__2(lean_object* x_1) { _start: { uint8_t x_2; @@ -6152,15 +6260,15 @@ x_2 = 0; return x_2; } } -static lean_object* _init_l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__1() { +static lean_object* _init_l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___lambda__2___boxed), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___lambda__2___boxed), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__2() { +static lean_object* _init_l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__2() { _start: { lean_object* x_1; @@ -6168,7 +6276,7 @@ x_1 = lean_mk_string_unchecked("unknown namespace '", 19, 19); return x_1; } } -static lean_object* _init_l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__3() { +static lean_object* _init_l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__3() { _start: { lean_object* x_1; @@ -6176,7 +6284,7 @@ x_1 = lean_mk_string_unchecked("'", 1, 1); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___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_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4(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; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; @@ -6228,17 +6336,17 @@ uint8_t x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_obje lean_dec(x_19); lean_free_object(x_14); x_21 = 1; -x_22 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__1; +x_22 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__1; x_23 = l_Lean_Name_toString(x_1, x_21, x_22); -x_24 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__2; +x_24 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__2; x_25 = lean_string_append(x_24, x_23); lean_dec(x_23); -x_26 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__3; +x_26 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__3; x_27 = lean_string_append(x_25, x_26); x_28 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_28, 0, x_27); x_29 = l_Lean_MessageData_ofFormat(x_28); -x_30 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_29, x_3, x_4, x_17); +x_30 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__7(x_29, x_3, x_4, x_17); x_31 = !lean_is_exclusive(x_30); if (x_31 == 0) { @@ -6300,17 +6408,17 @@ else uint8_t x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_dec(x_38); x_41 = 1; -x_42 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__1; +x_42 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__1; x_43 = l_Lean_Name_toString(x_1, x_41, x_42); -x_44 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__2; +x_44 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__2; x_45 = lean_string_append(x_44, x_43); lean_dec(x_43); -x_46 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__3; +x_46 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__3; x_47 = lean_string_append(x_45, x_46); x_48 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_48, 0, x_47); x_49 = l_Lean_MessageData_ofFormat(x_48); -x_50 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_49, x_3, x_4, x_36); +x_50 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__7(x_49, x_3, x_4, x_36); x_51 = lean_ctor_get(x_50, 0); lean_inc(x_51); x_52 = lean_ctor_get(x_50, 1); @@ -6427,7 +6535,7 @@ x_16 = lean_ctor_get(x_2, 6); lean_dec(x_16); lean_ctor_set(x_2, 6, x_14); x_17 = 0; -x_18 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3(x_5, x_17, x_2, x_3, x_13); +x_18 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4(x_5, x_17, x_2, x_3, x_13); return x_18; } else @@ -6466,7 +6574,7 @@ lean_ctor_set(x_29, 8, x_26); lean_ctor_set(x_29, 9, x_27); lean_ctor_set_uint8(x_29, sizeof(void*)*10, x_28); x_30 = 0; -x_31 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3(x_5, x_30, x_29, x_3, x_13); +x_31 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4(x_5, x_30, x_29, x_3, x_13); return x_31; } } @@ -6481,7 +6589,7 @@ return x_33; } } } -LEAN_EXPORT lean_object* l_Lean_resolveGlobalName___at_Lean_Elab_Command_elabExport___spec__9(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_resolveGlobalName___at_Lean_Elab_Command_elabExport___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; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; @@ -6535,7 +6643,7 @@ return x_23; } } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__12(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_throwError___at_Lean_Elab_Command_elabExport___spec__13(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; @@ -6607,7 +6715,7 @@ return x_22; } } } -static lean_object* _init_l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__11___closed__1() { +static lean_object* _init_l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__12___closed__1() { _start: { lean_object* x_1; @@ -6615,44 +6723,44 @@ x_1 = lean_mk_string_unchecked("unknown constant '", 18, 18); return x_1; } } -static lean_object* _init_l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__11___closed__2() { +static lean_object* _init_l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__12___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__11___closed__1; +x_1 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__12___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__11___closed__3() { +static lean_object* _init_l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__12___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__3; +x_1 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__3; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___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_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__12(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; x_6 = lean_box(0); x_7 = l_Lean_Expr_const___override(x_1, x_6); x_8 = l_Lean_MessageData_ofExpr(x_7); -x_9 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__11___closed__2; +x_9 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__12___closed__2; x_10 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_10, 0, x_9); lean_ctor_set(x_10, 1, x_8); -x_11 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__11___closed__3; +x_11 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__12___closed__3; x_12 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_12, 0, x_10); lean_ctor_set(x_12, 1, x_11); -x_13 = l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__12(x_12, x_2, x_3, x_4, x_5); +x_13 = l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__13(x_12, x_2, x_3, x_4, x_5); return x_13; } } -LEAN_EXPORT lean_object* l_Lean_filterFieldList___at_Lean_Elab_Command_elabExport___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_EXPORT lean_object* l_Lean_filterFieldList___at_Lean_Elab_Command_elabExport___spec__11___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; lean_object* x_9; @@ -6663,7 +6771,7 @@ lean_ctor_set(x_9, 1, x_7); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_filterFieldList___at_Lean_Elab_Command_elabExport___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_EXPORT lean_object* l_Lean_filterFieldList___at_Lean_Elab_Command_elabExport___spec__11(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; lean_object* x_8; uint8_t x_9; @@ -6675,14 +6783,14 @@ if (x_9 == 0) lean_object* x_10; lean_object* x_11; lean_dec(x_1); x_10 = lean_box(0); -x_11 = l_Lean_filterFieldList___at_Lean_Elab_Command_elabExport___spec__10___lambda__1(x_8, x_7, x_10, x_3, x_4, x_5, x_6); +x_11 = l_Lean_filterFieldList___at_Lean_Elab_Command_elabExport___spec__11___lambda__1(x_8, x_7, x_10, x_3, x_4, x_5, x_6); return x_11; } else { lean_object* x_12; uint8_t x_13; lean_dec(x_8); -x_12 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__11(x_1, x_3, x_4, x_5, x_6); +x_12 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__12(x_1, x_3, x_4, x_5, x_6); x_13 = !lean_is_exclusive(x_12); if (x_13 == 0) { @@ -6704,22 +6812,22 @@ return x_16; } } } -LEAN_EXPORT lean_object* l___private_Lean_ResolveName_0__Lean_resolveGlobalConstCore___at_Lean_Elab_Command_elabExport___spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l___private_Lean_ResolveName_0__Lean_resolveGlobalConstCore___at_Lean_Elab_Command_elabExport___spec__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_inc(x_1); -x_6 = l_Lean_resolveGlobalName___at_Lean_Elab_Command_elabExport___spec__9(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Lean_resolveGlobalName___at_Lean_Elab_Command_elabExport___spec__10(x_1, x_2, x_3, x_4, x_5); x_7 = lean_ctor_get(x_6, 0); lean_inc(x_7); x_8 = lean_ctor_get(x_6, 1); lean_inc(x_8); lean_dec(x_6); -x_9 = l_Lean_filterFieldList___at_Lean_Elab_Command_elabExport___spec__10(x_1, x_7, x_2, x_3, x_4, x_8); +x_9 = l_Lean_filterFieldList___at_Lean_Elab_Command_elabExport___spec__11(x_1, x_7, x_2, x_3, x_4, x_8); return x_9; } } -LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_Command_elabExport___spec__14(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_Command_elabExport___spec__15(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_2) == 0) @@ -6770,7 +6878,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabExport___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_throwError___at_Lean_Elab_Command_elabExport___spec__16(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; @@ -6842,7 +6950,7 @@ return x_22; } } } -LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_Command_elabExport___spec__16(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_Command_elabExport___spec__17(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_2) == 0) @@ -6893,7 +7001,7 @@ goto _start; } } } -static lean_object* _init_l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__13___closed__1() { +static lean_object* _init_l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__14___closed__1() { _start: { lean_object* x_1; @@ -6901,7 +7009,7 @@ x_1 = lean_mk_string_unchecked("ambiguous identifier '", 22, 22); return x_1; } } -static lean_object* _init_l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__13___closed__2() { +static lean_object* _init_l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__14___closed__2() { _start: { lean_object* x_1; @@ -6909,7 +7017,7 @@ x_1 = lean_mk_string_unchecked("', possible interpretations: ", 29, 29); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___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_EXPORT lean_object* l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___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) { _start: { if (lean_obj_tag(x_2) == 0) @@ -6919,12 +7027,12 @@ x_7 = lean_box(0); x_8 = l_Lean_Expr_const___override(x_1, x_7); x_9 = lean_expr_dbg_to_string(x_8); lean_dec(x_8); -x_10 = l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__13___closed__1; +x_10 = l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__14___closed__1; x_11 = lean_string_append(x_10, x_9); lean_dec(x_9); -x_12 = l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__13___closed__2; +x_12 = l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__14___closed__2; x_13 = lean_string_append(x_11, x_12); -x_14 = l_List_mapTR_loop___at_Lean_Elab_Command_elabExport___spec__14(x_7, x_2, x_7); +x_14 = l_List_mapTR_loop___at_Lean_Elab_Command_elabExport___spec__15(x_7, x_2, x_7); x_15 = l_List_toString___at_Lean_ensureNoOverload___spec__2(x_14); lean_dec(x_14); x_16 = lean_string_append(x_13, x_15); @@ -6934,7 +7042,7 @@ x_18 = lean_string_append(x_16, x_17); x_19 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_19, 0, x_18); x_20 = l_Lean_MessageData_ofFormat(x_19); -x_21 = l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__15(x_20, x_3, x_4, x_5, x_6); +x_21 = l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__16(x_20, x_3, x_4, x_5, x_6); return x_21; } else @@ -6976,12 +7084,12 @@ x_27 = lean_box(0); x_28 = l_Lean_Expr_const___override(x_1, x_27); x_29 = lean_expr_dbg_to_string(x_28); lean_dec(x_28); -x_30 = l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__13___closed__1; +x_30 = l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__14___closed__1; x_31 = lean_string_append(x_30, x_29); lean_dec(x_29); -x_32 = l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__13___closed__2; +x_32 = l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__14___closed__2; x_33 = lean_string_append(x_31, x_32); -x_34 = l_List_mapTR_loop___at_Lean_Elab_Command_elabExport___spec__16(x_27, x_2, x_27); +x_34 = l_List_mapTR_loop___at_Lean_Elab_Command_elabExport___spec__17(x_27, x_2, x_27); x_35 = l_List_toString___at_Lean_ensureNoOverload___spec__2(x_34); lean_dec(x_34); x_36 = lean_string_append(x_33, x_35); @@ -6991,18 +7099,18 @@ x_38 = lean_string_append(x_36, x_37); x_39 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_39, 0, x_38); x_40 = l_Lean_MessageData_ofFormat(x_39); -x_41 = l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__15(x_40, x_3, x_4, x_5, x_6); +x_41 = l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__16(x_40, x_3, x_4, x_5, x_6); return x_41; } } } } -LEAN_EXPORT lean_object* l_Lean_resolveGlobalConstNoOverloadCore___at_Lean_Elab_Command_elabExport___spec__7(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_resolveGlobalConstNoOverloadCore___at_Lean_Elab_Command_elabExport___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_inc(x_1); -x_6 = l___private_Lean_ResolveName_0__Lean_resolveGlobalConstCore___at_Lean_Elab_Command_elabExport___spec__8(x_1, x_2, x_3, x_4, x_5); +x_6 = l___private_Lean_ResolveName_0__Lean_resolveGlobalConstCore___at_Lean_Elab_Command_elabExport___spec__9(x_1, x_2, 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; @@ -7011,7 +7119,7 @@ lean_inc(x_7); x_8 = lean_ctor_get(x_6, 1); lean_inc(x_8); lean_dec(x_6); -x_9 = l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__13(x_1, x_7, x_2, x_3, x_4, x_8); +x_9 = l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__14(x_1, x_7, x_2, x_3, x_4, x_8); return x_9; } else @@ -7039,7 +7147,7 @@ return x_13; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_OpenDecl_resolveId___at_Lean_Elab_Command_elabExport___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Elab_OpenDecl_resolveId___at_Lean_Elab_Command_elabExport___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; @@ -7075,7 +7183,7 @@ lean_object* x_20; lean_object* x_21; x_20 = lean_ctor_get(x_4, 6); lean_dec(x_20); lean_ctor_set(x_4, 6, x_18); -x_21 = l_Lean_resolveGlobalConstNoOverloadCore___at_Lean_Elab_Command_elabExport___spec__7(x_8, x_3, x_4, x_5, x_17); +x_21 = l_Lean_resolveGlobalConstNoOverloadCore___at_Lean_Elab_Command_elabExport___spec__8(x_8, x_3, x_4, x_5, x_17); lean_dec(x_4); return x_21; } @@ -7114,7 +7222,7 @@ lean_ctor_set(x_32, 7, x_28); lean_ctor_set(x_32, 8, x_29); lean_ctor_set(x_32, 9, x_30); lean_ctor_set_uint8(x_32, sizeof(void*)*10, x_31); -x_33 = l_Lean_resolveGlobalConstNoOverloadCore___at_Lean_Elab_Command_elabExport___spec__7(x_8, x_3, x_32, x_5, x_17); +x_33 = l_Lean_resolveGlobalConstNoOverloadCore___at_Lean_Elab_Command_elabExport___spec__8(x_8, x_3, x_32, x_5, x_17); lean_dec(x_32); return x_33; } @@ -7200,7 +7308,7 @@ 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_uint8(x_53, sizeof(void*)*10, x_51); -x_54 = l_Lean_resolveGlobalConstNoOverloadCore___at_Lean_Elab_Command_elabExport___spec__7(x_8, x_3, x_53, x_5, x_40); +x_54 = l_Lean_resolveGlobalConstNoOverloadCore___at_Lean_Elab_Command_elabExport___spec__8(x_8, x_3, x_53, x_5, x_40); lean_dec(x_53); return x_54; } @@ -7216,7 +7324,7 @@ return x_55; } } } -LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Command_elabExport___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_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Command_elabExport___spec__18(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { if (lean_obj_tag(x_2) == 0) @@ -7243,7 +7351,7 @@ lean_object* x_12; lean_object* x_13; lean_object* x_14; x_12 = lean_ctor_get(x_3, 0); x_13 = lean_ctor_get(x_3, 1); lean_inc(x_5); -x_14 = l_Lean_Elab_OpenDecl_resolveId___at_Lean_Elab_Command_elabExport___spec__6(x_9, x_1, x_4, x_5, x_6, x_7); +x_14 = l_Lean_Elab_OpenDecl_resolveId___at_Lean_Elab_Command_elabExport___spec__7(x_9, x_1, 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; @@ -7331,7 +7439,7 @@ lean_inc(x_32); lean_inc(x_31); lean_dec(x_3); lean_inc(x_5); -x_33 = l_Lean_Elab_OpenDecl_resolveId___at_Lean_Elab_Command_elabExport___spec__6(x_9, x_1, x_4, x_5, x_6, x_7); +x_33 = l_Lean_Elab_OpenDecl_resolveId___at_Lean_Elab_Command_elabExport___spec__7(x_9, x_1, x_4, x_5, x_6, x_7); if (lean_obj_tag(x_33) == 0) { lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; @@ -7399,7 +7507,7 @@ return x_46; } } } -LEAN_EXPORT lean_object* l_Lean_getRefPos___at_Lean_Elab_Command_elabExport___spec__20___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_getRefPos___at_Lean_Elab_Command_elabExport___spec__21___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; uint8_t x_5; @@ -7463,15 +7571,15 @@ return x_18; } } } -LEAN_EXPORT lean_object* l_Lean_getRefPos___at_Lean_Elab_Command_elabExport___spec__20(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_getRefPos___at_Lean_Elab_Command_elabExport___spec__21(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_getRefPos___at_Lean_Elab_Command_elabExport___spec__20___rarg___boxed), 3, 0); +x_2 = lean_alloc_closure((void*)(l_Lean_getRefPos___at_Lean_Elab_Command_elabExport___spec__21___rarg___boxed), 3, 0); return x_2; } } -static lean_object* _init_l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__1() { +static lean_object* _init_l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__1() { _start: { lean_object* x_1; @@ -7479,16 +7587,16 @@ x_1 = lean_mk_string_unchecked(":", 1, 1); return x_1; } } -static lean_object* _init_l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__2() { +static lean_object* _init_l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__1; +x_1 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__3() { +static lean_object* _init_l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__3() { _start: { lean_object* x_1; @@ -7496,20 +7604,20 @@ x_1 = lean_mk_string_unchecked(" ", 1, 1); return x_1; } } -static lean_object* _init_l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__4() { +static lean_object* _init_l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__3; +x_1 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__3; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; uint8_t x_7; -x_6 = l_Lean_getRefPos___at_Lean_Elab_Command_elabExport___spec__20___rarg(x_3, x_4, x_5); +x_6 = l_Lean_getRefPos___at_Lean_Elab_Command_elabExport___spec__21___rarg(x_3, x_4, x_5); x_7 = !lean_is_exclusive(x_6); if (x_7 == 0) { @@ -7556,7 +7664,7 @@ x_21 = l_Lean_Elab_Command_elabModuleDoc___closed__4; x_22 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_22, 0, x_21); lean_ctor_set(x_22, 1, x_20); -x_23 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__2; +x_23 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__2; x_24 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_24, 0, x_22); lean_ctor_set(x_24, 1, x_23); @@ -7570,7 +7678,7 @@ x_28 = l_Lean_MessageData_ofFormat(x_27); x_29 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_29, 0, x_24); lean_ctor_set(x_29, 1, x_28); -x_30 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__4; +x_30 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__4; x_31 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_31, 0, x_29); lean_ctor_set(x_31, 1, x_30); @@ -7621,7 +7729,7 @@ x_44 = l_Lean_Elab_Command_elabModuleDoc___closed__4; x_45 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_45, 0, x_44); lean_ctor_set(x_45, 1, x_43); -x_46 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__2; +x_46 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__2; x_47 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_47, 0, x_45); lean_ctor_set(x_47, 1, x_46); @@ -7635,7 +7743,7 @@ x_51 = l_Lean_MessageData_ofFormat(x_50); x_52 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_52, 0, x_47); lean_ctor_set(x_52, 1, x_51); -x_53 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__4; +x_53 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__4; x_54 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_54, 0, x_52); lean_ctor_set(x_54, 1, x_53); @@ -7721,7 +7829,7 @@ x_75 = l_Lean_Elab_Command_elabModuleDoc___closed__4; x_76 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_76, 0, x_75); lean_ctor_set(x_76, 1, x_74); -x_77 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__2; +x_77 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__2; x_78 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_78, 0, x_76); lean_ctor_set(x_78, 1, x_77); @@ -7735,7 +7843,7 @@ x_82 = l_Lean_MessageData_ofFormat(x_81); x_83 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_83, 0, x_78); lean_ctor_set(x_83, 1, x_82); -x_84 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__4; +x_84 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__4; x_85 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_85, 0, x_83); lean_ctor_set(x_85, 1, x_84); @@ -7767,7 +7875,7 @@ return x_91; } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabExport___spec__21(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_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabExport___spec__22(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) { _start: { uint8_t x_8; @@ -7788,7 +7896,7 @@ x_10 = lean_array_uget(x_3, x_2); x_11 = lean_unsigned_to_nat(0u); x_12 = lean_array_uset(x_3, x_2, x_11); lean_inc(x_5); -x_13 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19(x_10, x_4, x_5, x_6, x_7); +x_13 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20(x_10, x_4, x_5, x_6, x_7); x_14 = lean_ctor_get(x_13, 0); lean_inc(x_14); x_15 = lean_ctor_get(x_13, 1); @@ -7804,7 +7912,7 @@ goto _start; } } } -static lean_object* _init_l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__18___closed__1() { +static lean_object* _init_l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__19___closed__1() { _start: { lean_object* x_1; @@ -7812,23 +7920,23 @@ x_1 = lean_mk_string_unchecked(", errors ", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__18___closed__2() { +static lean_object* _init_l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__19___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__18___closed__1; +x_1 = l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__19___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__18(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__19(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { size_t x_7; size_t x_8; lean_object* x_9; uint8_t x_10; x_7 = lean_array_size(x_2); x_8 = 0; lean_inc(x_4); -x_9 = l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabExport___spec__21(x_7, x_8, x_2, x_3, x_4, x_5, x_6); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabExport___spec__22(x_7, x_8, x_2, x_3, x_4, x_5, x_6); x_10 = !lean_is_exclusive(x_9); if (x_10 == 0) { @@ -7839,7 +7947,7 @@ x_13 = l_Lean_Elab_Command_elabModuleDoc___closed__4; lean_ctor_set_tag(x_9, 7); lean_ctor_set(x_9, 1, x_1); lean_ctor_set(x_9, 0, x_13); -x_14 = l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__18___closed__2; +x_14 = l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__19___closed__2; x_15 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_15, 0, x_9); lean_ctor_set(x_15, 1, x_14); @@ -7850,7 +7958,7 @@ lean_ctor_set(x_17, 1, x_16); x_18 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_18, 0, x_17); lean_ctor_set(x_18, 1, x_13); -x_19 = l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__12(x_18, x_3, x_4, x_5, x_12); +x_19 = l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__13(x_18, x_3, x_4, x_5, x_12); lean_dec(x_4); return x_19; } @@ -7866,7 +7974,7 @@ x_22 = l_Lean_Elab_Command_elabModuleDoc___closed__4; x_23 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_23, 0, x_22); lean_ctor_set(x_23, 1, x_1); -x_24 = l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__18___closed__2; +x_24 = l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__19___closed__2; x_25 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_25, 0, x_23); lean_ctor_set(x_25, 1, x_24); @@ -7877,31 +7985,31 @@ lean_ctor_set(x_27, 1, x_26); 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_throwError___at_Lean_Elab_Command_elabExport___spec__12(x_28, x_3, x_4, x_5, x_21); +x_29 = l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__13(x_28, x_3, x_4, x_5, x_21); lean_dec(x_4); return x_29; } } } -static lean_object* _init_l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___lambda__1___closed__1() { +static lean_object* _init_l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___lambda__1___closed__1() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__13___closed__1; +x_1 = l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__14___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___lambda__1___closed__2() { +static lean_object* _init_l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___lambda__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__13___closed__2; +x_1 = l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__14___closed__2; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___lambda__1(lean_object* x_1, lean_object* x_2, lean_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_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___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) { _start: { lean_object* x_9; lean_object* x_10; uint8_t x_11; @@ -7914,11 +8022,11 @@ lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean lean_dec(x_9); x_12 = l_Lean_Syntax_getId(x_2); x_13 = l_Lean_MessageData_ofName(x_12); -x_14 = l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___lambda__1___closed__1; +x_14 = l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___lambda__1___closed__1; x_15 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_15, 0, x_14); lean_ctor_set(x_15, 1, x_13); -x_16 = l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___lambda__1___closed__2; +x_16 = l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___lambda__1___closed__2; x_17 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_17, 0, x_15); lean_ctor_set(x_17, 1, x_16); @@ -7950,7 +8058,7 @@ lean_object* x_32; lean_object* x_33; x_32 = lean_ctor_get(x_6, 6); lean_dec(x_32); lean_ctor_set(x_6, 6, x_30); -x_33 = l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__15(x_26, x_5, x_6, x_7, x_29); +x_33 = l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__16(x_26, x_5, x_6, x_7, x_29); lean_dec(x_6); return x_33; } @@ -7989,7 +8097,7 @@ lean_ctor_set(x_44, 7, x_40); lean_ctor_set(x_44, 8, x_41); lean_ctor_set(x_44, 9, x_42); lean_ctor_set_uint8(x_44, sizeof(void*)*10, x_43); -x_45 = l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__15(x_26, x_5, x_44, x_7, x_29); +x_45 = l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__16(x_26, x_5, x_44, x_7, x_29); lean_dec(x_44); return x_45; } @@ -8026,7 +8134,7 @@ return x_52; } } } -static lean_object* _init_l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___closed__1() { +static lean_object* _init_l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___closed__1() { _start: { lean_object* x_1; lean_object* x_2; @@ -8037,7 +8145,7 @@ lean_ctor_set(x_2, 1, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___closed__2() { +static lean_object* _init_l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___closed__2() { _start: { lean_object* x_1; @@ -8045,34 +8153,34 @@ x_1 = lean_mk_string_unchecked("failed to open", 14, 14); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___closed__3() { +static lean_object* _init_l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___closed__2; +x_1 = l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___closed__2; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___closed__4() { +static lean_object* _init_l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___closed__3; +x_1 = l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___closed__3; x_2 = l_Lean_MessageData_ofFormat(x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___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: { lean_object* x_7; lean_object* x_8; lean_object* x_9; x_7 = lean_box(0); -x_8 = l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___closed__1; +x_8 = l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___closed__1; lean_inc(x_4); lean_inc(x_1); -x_9 = l_List_forIn_loop___at_Lean_Elab_Command_elabExport___spec__17(x_2, x_1, x_8, x_3, x_4, x_5, x_6); +x_9 = l_List_forIn_loop___at_Lean_Elab_Command_elabExport___spec__18(x_2, x_1, x_8, x_3, x_4, x_5, x_6); if (lean_obj_tag(x_9) == 0) { lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; @@ -8098,7 +8206,7 @@ lean_object* x_18; lean_object* x_19; lean_dec(x_14); lean_dec(x_12); x_18 = lean_box(0); -x_19 = l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___lambda__1(x_13, x_2, x_7, x_18, x_3, x_4, x_5, x_11); +x_19 = l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___lambda__1(x_13, x_2, x_7, x_18, x_3, x_4, x_5, x_11); return x_19; } else @@ -8143,8 +8251,8 @@ lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; x_28 = lean_ctor_get(x_4, 6); lean_dec(x_28); lean_ctor_set(x_4, 6, x_26); -x_29 = l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___closed__4; -x_30 = l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__18(x_29, x_12, x_3, x_4, x_5, x_25); +x_29 = l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___closed__4; +x_30 = l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__19(x_29, x_12, x_3, x_4, x_5, x_25); x_31 = !lean_is_exclusive(x_30); if (x_31 == 0) { @@ -8199,8 +8307,8 @@ lean_ctor_set(x_45, 7, x_41); lean_ctor_set(x_45, 8, x_42); lean_ctor_set(x_45, 9, x_43); lean_ctor_set_uint8(x_45, sizeof(void*)*10, x_44); -x_46 = l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___closed__4; -x_47 = l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__18(x_46, x_12, x_3, x_45, x_5, x_25); +x_46 = l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___closed__4; +x_47 = l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__19(x_46, x_12, x_3, x_45, x_5, x_25); x_48 = lean_ctor_get(x_47, 0); lean_inc(x_48); x_49 = lean_ctor_get(x_47, 1); @@ -8315,7 +8423,7 @@ return x_71; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_OpenDecl_resolveNameUsingNamespaces___at_Lean_Elab_Command_elabExport___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_Elab_OpenDecl_resolveNameUsingNamespaces___at_Lean_Elab_Command_elabExport___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; @@ -8346,7 +8454,7 @@ lean_inc(x_16); x_17 = lean_ctor_get(x_15, 1); lean_inc(x_17); lean_dec(x_15); -x_18 = l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5(x_1, x_2, x_16, x_3, x_4, x_17); +x_18 = l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6(x_1, x_2, x_16, x_3, x_4, x_17); if (lean_obj_tag(x_18) == 0) { lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; @@ -8422,7 +8530,7 @@ lean_inc(x_35); x_36 = lean_ctor_get(x_34, 1); lean_inc(x_36); lean_dec(x_34); -x_37 = l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5(x_1, x_2, x_35, x_3, x_4, x_36); +x_37 = l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6(x_1, x_2, x_35, x_3, x_4, x_36); if (lean_obj_tag(x_37) == 0) { lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; @@ -8480,72 +8588,318 @@ return x_47; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_addConstInfo___at_Lean_Elab_Command_elabExport___spec__22(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__26(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_7; -lean_inc(x_4); -x_7 = l_Lean_mkConstWithLevelParams___at_Lean_Elab_Command_expandDeclId___spec__8(x_2, x_4, x_5, x_6); -if (lean_obj_tag(x_7) == 0) -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_8 = lean_ctor_get(x_7, 0); +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_5 = l_Lean_Elab_Command_getRef(x_2, x_3, x_4); +x_6 = lean_ctor_get(x_5, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_5, 1); +lean_inc(x_7); +lean_dec(x_5); +x_8 = lean_ctor_get(x_2, 4); lean_inc(x_8); -x_9 = lean_ctor_get(x_7, 1); -lean_inc(x_9); -lean_dec(x_7); -x_10 = lean_box(0); -x_11 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_11, 0, x_10); -lean_ctor_set(x_11, 1, x_1); -x_12 = l_Lean_LocalContext_empty; -x_13 = 0; -x_14 = lean_alloc_ctor(0, 4, 1); -lean_ctor_set(x_14, 0, x_11); -lean_ctor_set(x_14, 1, x_12); -lean_ctor_set(x_14, 2, x_3); -lean_ctor_set(x_14, 3, x_8); -lean_ctor_set_uint8(x_14, sizeof(void*)*4, x_13); -x_15 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_15, 0, x_14); -x_16 = l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_expandDeclId___spec__11(x_15, x_4, x_5, x_9); -lean_dec(x_4); -return x_16; -} -else +lean_inc(x_8); +x_9 = l_Lean_Elab_getBetterRef(x_6, x_8); +lean_dec(x_6); +x_10 = l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1(x_1, x_2, x_3, x_7); +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) { -uint8_t x_17; -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_17 = !lean_is_exclusive(x_7); -if (x_17 == 0) +lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_12 = lean_ctor_get(x_10, 0); +x_13 = lean_ctor_get(x_10, 1); +x_14 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_12, x_8, x_2, x_3, x_13); +lean_dec(x_2); +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 0) { -return x_7; +lean_object* x_16; +x_16 = lean_ctor_get(x_14, 0); +lean_ctor_set(x_10, 1, x_16); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set_tag(x_14, 1); +lean_ctor_set(x_14, 0, x_10); +return x_14; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_7, 0); -x_19 = lean_ctor_get(x_7, 1); -lean_inc(x_19); +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_14, 0); +x_18 = lean_ctor_get(x_14, 1); lean_inc(x_18); -lean_dec(x_7); -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_inc(x_17); +lean_dec(x_14); +lean_ctor_set(x_10, 1, x_17); +lean_ctor_set(x_10, 0, x_9); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_10); +lean_ctor_set(x_19, 1, x_18); +return x_19; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabExport___spec__23___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; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_9 = l_Lean_Name_append(x_1, x_2); -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_9); +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_20 = lean_ctor_get(x_10, 0); +x_21 = lean_ctor_get(x_10, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_10); +x_22 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_20, x_8, x_2, x_3, x_21); +lean_dec(x_2); +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +if (lean_is_exclusive(x_22)) { + lean_ctor_release(x_22, 0); + lean_ctor_release(x_22, 1); + x_25 = x_22; +} else { + lean_dec_ref(x_22); + x_25 = lean_box(0); +} +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_9); +lean_ctor_set(x_26, 1, x_23); +if (lean_is_scalar(x_25)) { + x_27 = lean_alloc_ctor(1, 2, 0); +} else { + x_27 = x_25; + lean_ctor_set_tag(x_27, 1); +} +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_24); +return x_27; +} +} +} +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at_Lean_Elab_Command_elabExport___spec__25(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_3, x_4); +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; +x_7 = lean_ctor_get(x_5, 0); +x_8 = lean_ctor_get(x_5, 1); +x_9 = lean_ctor_get(x_7, 0); +lean_inc(x_9); +lean_dec(x_7); +lean_inc(x_1); +x_10 = lean_environment_find(x_9, x_1); +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; +lean_free_object(x_5); +x_11 = lean_box(0); +x_12 = l_Lean_Expr_const___override(x_1, x_11); +x_13 = l_Lean_MessageData_ofExpr(x_12); +x_14 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__12___closed__2; +x_15 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_13); +x_16 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__12___closed__3; +x_17 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_17, 0, x_15); +lean_ctor_set(x_17, 1, x_16); +x_18 = l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__26(x_17, x_2, x_3, x_8); +return x_18; +} +else +{ +lean_object* x_19; +lean_dec(x_2); +lean_dec(x_1); +x_19 = lean_ctor_get(x_10, 0); +lean_inc(x_19); +lean_dec(x_10); +lean_ctor_set(x_5, 0, x_19); +return x_5; +} +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_20 = lean_ctor_get(x_5, 0); +x_21 = lean_ctor_get(x_5, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_5); +x_22 = lean_ctor_get(x_20, 0); +lean_inc(x_22); +lean_dec(x_20); +lean_inc(x_1); +x_23 = lean_environment_find(x_22, x_1); +if (lean_obj_tag(x_23) == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_24 = lean_box(0); +x_25 = l_Lean_Expr_const___override(x_1, x_24); +x_26 = l_Lean_MessageData_ofExpr(x_25); +x_27 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__12___closed__2; +x_28 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_26); +x_29 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__12___closed__3; +x_30 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +x_31 = l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__26(x_30, x_2, x_3, x_21); +return x_31; +} +else +{ +lean_object* x_32; lean_object* x_33; +lean_dec(x_2); +lean_dec(x_1); +x_32 = lean_ctor_get(x_23, 0); +lean_inc(x_32); +lean_dec(x_23); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_21); +return x_33; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_mkConstWithLevelParams___at_Lean_Elab_Command_elabExport___spec__24(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +lean_inc(x_1); +x_5 = l_Lean_getConstInfo___at_Lean_Elab_Command_elabExport___spec__25(x_1, x_2, x_3, x_4); +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +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; +x_7 = lean_ctor_get(x_5, 0); +x_8 = l_Lean_ConstantInfo_levelParams(x_7); +lean_dec(x_7); +x_9 = lean_box(0); +x_10 = l_List_mapTR_loop___at_Lean_mkConstWithLevelParams___spec__1(x_8, x_9); +x_11 = l_Lean_Expr_const___override(x_1, 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; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_12 = lean_ctor_get(x_5, 0); +x_13 = lean_ctor_get(x_5, 1); +lean_inc(x_13); +lean_inc(x_12); +lean_dec(x_5); +x_14 = l_Lean_ConstantInfo_levelParams(x_12); +lean_dec(x_12); +x_15 = lean_box(0); +x_16 = l_List_mapTR_loop___at_Lean_mkConstWithLevelParams___spec__1(x_14, x_15); +x_17 = l_Lean_Expr_const___override(x_1, x_16); +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set(x_18, 1, x_13); +return x_18; +} +} +else +{ +uint8_t x_19; +lean_dec(x_1); +x_19 = !lean_is_exclusive(x_5); +if (x_19 == 0) +{ +return x_5; +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_5, 0); +x_21 = lean_ctor_get(x_5, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_5); +x_22 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_22, 0, x_20); +lean_ctor_set(x_22, 1, x_21); +return x_22; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_addConstInfo___at_Lean_Elab_Command_elabExport___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) { +_start: +{ +lean_object* x_7; +lean_inc(x_4); +x_7 = l_Lean_mkConstWithLevelParams___at_Lean_Elab_Command_elabExport___spec__24(x_2, x_4, x_5, x_6); +if (lean_obj_tag(x_7) == 0) +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_8 = lean_ctor_get(x_7, 0); +lean_inc(x_8); +x_9 = lean_ctor_get(x_7, 1); +lean_inc(x_9); +lean_dec(x_7); +x_10 = lean_box(0); +x_11 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_11, 0, x_10); +lean_ctor_set(x_11, 1, x_1); +x_12 = l_Lean_LocalContext_empty; +x_13 = 0; +x_14 = lean_alloc_ctor(0, 4, 1); +lean_ctor_set(x_14, 0, x_11); +lean_ctor_set(x_14, 1, x_12); +lean_ctor_set(x_14, 2, x_3); +lean_ctor_set(x_14, 3, x_8); +lean_ctor_set_uint8(x_14, sizeof(void*)*4, x_13); +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_14); +x_16 = l_Lean_Elab_pushInfoLeaf___at_Lean_withSetOptionIn___spec__3(x_15, x_4, x_5, x_9); +lean_dec(x_4); +return x_16; +} +else +{ +uint8_t x_17; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_17 = !lean_is_exclusive(x_7); +if (x_17 == 0) +{ +return x_7; +} +else +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_7, 0); +x_19 = lean_ctor_get(x_7, 1); +lean_inc(x_19); +lean_inc(x_18); +lean_dec(x_7); +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_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabExport___spec__27___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_9 = l_Lean_Name_append(x_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_3); x_11 = lean_array_push(x_4, x_10); x_12 = lean_alloc_ctor(1, 1, 0); @@ -8556,7 +8910,7 @@ lean_ctor_set(x_13, 1, x_8); return x_13; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabExport___spec__23(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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabExport___spec__27(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) { _start: { uint8_t x_10; @@ -8579,7 +8933,7 @@ x_12 = lean_array_uget(x_3, x_5); x_13 = l_Lean_Syntax_getId(x_12); lean_inc(x_7); lean_inc(x_1); -x_14 = l_Lean_Elab_OpenDecl_resolveNameUsingNamespaces___at_Lean_Elab_Command_elabExport___spec__4(x_1, x_12, x_7, x_8, x_9); +x_14 = l_Lean_Elab_OpenDecl_resolveNameUsingNamespaces___at_Lean_Elab_Command_elabExport___spec__5(x_1, x_12, x_7, x_8, x_9); if (lean_obj_tag(x_14) == 0) { lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; @@ -8605,7 +8959,7 @@ lean_inc(x_21); lean_dec(x_17); x_22 = lean_box(0); lean_inc(x_2); -x_23 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabExport___spec__23___lambda__1(x_2, x_13, x_15, x_6, x_22, x_7, x_8, x_21); +x_23 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabExport___spec__27___lambda__1(x_2, x_13, x_15, x_6, x_22, x_7, x_8, x_21); x_24 = lean_ctor_get(x_23, 0); lean_inc(x_24); x_25 = lean_ctor_get(x_23, 1); @@ -8630,7 +8984,7 @@ lean_dec(x_17); x_31 = lean_box(0); lean_inc(x_7); lean_inc(x_15); -x_32 = l_Lean_Elab_addConstInfo___at_Lean_Elab_Command_elabExport___spec__22(x_12, x_15, x_31, x_7, x_8, x_30); +x_32 = l_Lean_Elab_addConstInfo___at_Lean_Elab_Command_elabExport___spec__23(x_12, x_15, x_31, x_7, x_8, x_30); 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; size_t x_39; size_t x_40; @@ -8640,7 +8994,7 @@ x_34 = lean_ctor_get(x_32, 1); lean_inc(x_34); lean_dec(x_32); lean_inc(x_2); -x_35 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabExport___spec__23___lambda__1(x_2, x_13, x_15, x_6, x_33, x_7, x_8, x_34); +x_35 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabExport___spec__27___lambda__1(x_2, x_13, x_15, x_6, x_33, x_7, x_8, x_34); lean_dec(x_33); x_36 = lean_ctor_get(x_35, 0); lean_inc(x_36); @@ -8718,7 +9072,7 @@ return x_49; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabExport___spec__24(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabExport___spec__28(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { uint8_t x_5; @@ -8752,7 +9106,7 @@ size_t x_8; size_t x_9; lean_object* x_10; lean_object* x_11; x_8 = lean_array_size(x_1); x_9 = 0; x_10 = l_Lean_resolveNamespace___at_Lean_Elab_Command_elabExport___spec__1___closed__4; -x_11 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabExport___spec__23(x_2, x_3, x_1, x_8, x_9, x_10, x_5, x_6, x_7); +x_11 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabExport___spec__27(x_2, x_3, x_1, x_8, x_9, 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; lean_object* x_15; lean_object* x_16; uint8_t x_17; @@ -8842,7 +9196,7 @@ else size_t x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; x_37 = lean_usize_of_nat(x_19); lean_dec(x_19); -x_38 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabExport___spec__24(x_12, x_9, x_37, x_18); +x_38 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabExport___spec__28(x_12, x_9, x_37, x_18); lean_dec(x_12); lean_ctor_set(x_15, 0, x_38); x_39 = lean_st_ref_set(x_6, x_15, x_16); @@ -8973,7 +9327,7 @@ else 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; x_70 = lean_usize_of_nat(x_54); lean_dec(x_54); -x_71 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabExport___spec__24(x_12, x_9, x_70, x_46); +x_71 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabExport___spec__28(x_12, x_9, x_70, x_46); lean_dec(x_12); x_72 = lean_alloc_ctor(0, 8, 0); lean_ctor_set(x_72, 0, x_71); @@ -9136,7 +9490,7 @@ lean_dec(x_20); lean_dec(x_14); lean_dec(x_12); x_25 = l_Lean_Elab_Command_elabExport___closed__4; -x_26 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_25, x_2, x_3, x_19); +x_26 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__7(x_25, x_2, x_3, x_19); x_27 = !lean_is_exclusive(x_26); if (x_27 == 0) { @@ -9190,7 +9544,7 @@ lean_dec(x_33); lean_dec(x_14); lean_dec(x_12); x_39 = l_Lean_Elab_Command_elabExport___closed__4; -x_40 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_39, x_2, x_3, x_32); +x_40 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__7(x_39, x_2, x_3, x_32); x_41 = lean_ctor_get(x_40, 0); lean_inc(x_41); x_42 = lean_ctor_get(x_40, 1); @@ -9241,6 +9595,15 @@ return x_48; } } } +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__3(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; +} +} LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabExport___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { @@ -9251,34 +9614,34 @@ lean_dec(x_1); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___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_EXPORT lean_object* l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___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) { _start: { lean_object* x_6; -x_6 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___lambda__1(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___lambda__1(x_1, x_2, x_3, x_4, x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___lambda__2___boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___lambda__2___boxed(lean_object* x_1) { _start: { uint8_t x_2; lean_object* x_3; -x_2 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___lambda__2(x_1); +x_2 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___lambda__2(x_1); lean_dec(x_1); x_3 = lean_box(x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___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_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___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_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3(x_1, x_6, x_3, x_4, x_5); +x_7 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4(x_1, x_6, x_3, x_4, x_5); lean_dec(x_4); return x_7; } @@ -9292,44 +9655,44 @@ lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_resolveGlobalName___at_Lean_Elab_Command_elabExport___spec__9___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_resolveGlobalName___at_Lean_Elab_Command_elabExport___spec__10___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_resolveGlobalName___at_Lean_Elab_Command_elabExport___spec__9(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Lean_resolveGlobalName___at_Lean_Elab_Command_elabExport___spec__10(x_1, x_2, x_3, x_4, x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__12___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_throwError___at_Lean_Elab_Command_elabExport___spec__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; -x_6 = l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__12(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__13(x_1, x_2, x_3, x_4, x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__11___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_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__12___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_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__11(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__12(x_1, x_2, x_3, x_4, x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_filterFieldList___at_Lean_Elab_Command_elabExport___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_EXPORT lean_object* l_Lean_filterFieldList___at_Lean_Elab_Command_elabExport___spec__11___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; -x_8 = l_Lean_filterFieldList___at_Lean_Elab_Command_elabExport___spec__10___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Lean_filterFieldList___at_Lean_Elab_Command_elabExport___spec__11___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); @@ -9337,113 +9700,113 @@ lean_dec(x_3); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_filterFieldList___at_Lean_Elab_Command_elabExport___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_EXPORT lean_object* l_Lean_filterFieldList___at_Lean_Elab_Command_elabExport___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; -x_7 = l_Lean_filterFieldList___at_Lean_Elab_Command_elabExport___spec__10(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Lean_filterFieldList___at_Lean_Elab_Command_elabExport___spec__11(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___private_Lean_ResolveName_0__Lean_resolveGlobalConstCore___at_Lean_Elab_Command_elabExport___spec__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l___private_Lean_ResolveName_0__Lean_resolveGlobalConstCore___at_Lean_Elab_Command_elabExport___spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; -x_6 = l___private_Lean_ResolveName_0__Lean_resolveGlobalConstCore___at_Lean_Elab_Command_elabExport___spec__8(x_1, x_2, x_3, x_4, x_5); +x_6 = l___private_Lean_ResolveName_0__Lean_resolveGlobalConstCore___at_Lean_Elab_Command_elabExport___spec__9(x_1, x_2, x_3, x_4, x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__15___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_throwError___at_Lean_Elab_Command_elabExport___spec__16___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_throwError___at_Lean_Elab_Command_elabExport___spec__15(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__16(x_1, x_2, x_3, x_4, x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___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_EXPORT lean_object* l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___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) { _start: { lean_object* x_7; -x_7 = l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__13(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__14(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_resolveGlobalConstNoOverloadCore___at_Lean_Elab_Command_elabExport___spec__7___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_resolveGlobalConstNoOverloadCore___at_Lean_Elab_Command_elabExport___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_resolveGlobalConstNoOverloadCore___at_Lean_Elab_Command_elabExport___spec__7(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Lean_resolveGlobalConstNoOverloadCore___at_Lean_Elab_Command_elabExport___spec__8(x_1, x_2, x_3, x_4, x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Elab_OpenDecl_resolveId___at_Lean_Elab_Command_elabExport___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Elab_OpenDecl_resolveId___at_Lean_Elab_Command_elabExport___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_7; -x_7 = l_Lean_Elab_OpenDecl_resolveId___at_Lean_Elab_Command_elabExport___spec__6(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Lean_Elab_OpenDecl_resolveId___at_Lean_Elab_Command_elabExport___spec__7(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_5); lean_dec(x_3); lean_dec(x_2); return x_7; } } -LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Command_elabExport___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_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Command_elabExport___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) { _start: { lean_object* x_8; -x_8 = l_List_forIn_loop___at_Lean_Elab_Command_elabExport___spec__17(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_List_forIn_loop___at_Lean_Elab_Command_elabExport___spec__18(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_6); lean_dec(x_4); lean_dec(x_1); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_getRefPos___at_Lean_Elab_Command_elabExport___spec__20___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_getRefPos___at_Lean_Elab_Command_elabExport___spec__21___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_Command_elabExport___spec__20___rarg(x_1, x_2, x_3); +x_4 = l_Lean_getRefPos___at_Lean_Elab_Command_elabExport___spec__21___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_Command_elabExport___spec__20___boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_getRefPos___at_Lean_Elab_Command_elabExport___spec__21___boxed(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l_Lean_getRefPos___at_Lean_Elab_Command_elabExport___spec__20(x_1); +x_2 = l_Lean_getRefPos___at_Lean_Elab_Command_elabExport___spec__21(x_1); lean_dec(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___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_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20(x_1, x_2, x_3, x_4, x_5); lean_dec(x_4); lean_dec(x_2); return x_6; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabExport___spec__21___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabExport___spec__22___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { size_t x_8; size_t x_9; lean_object* x_10; @@ -9451,27 +9814,27 @@ x_8 = lean_unbox_usize(x_1); lean_dec(x_1); x_9 = lean_unbox_usize(x_2); lean_dec(x_2); -x_10 = l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabExport___spec__21(x_8, x_9, x_3, x_4, x_5, x_6, x_7); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabExport___spec__22(x_8, x_9, x_3, x_4, x_5, x_6, x_7); lean_dec(x_6); lean_dec(x_4); return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__18___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___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) { _start: { lean_object* x_7; -x_7 = l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__18(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__19(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_5); lean_dec(x_3); return x_7; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___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) { _start: { lean_object* x_9; -x_9 = l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___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_5); lean_dec(x_4); @@ -9479,48 +9842,75 @@ lean_dec(x_2); return x_9; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___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) { _start: { lean_object* x_7; -x_7 = l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_5); lean_dec(x_3); lean_dec(x_2); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_OpenDecl_resolveNameUsingNamespaces___at_Lean_Elab_Command_elabExport___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_Elab_OpenDecl_resolveNameUsingNamespaces___at_Lean_Elab_Command_elabExport___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_Lean_Elab_OpenDecl_resolveNameUsingNamespaces___at_Lean_Elab_Command_elabExport___spec__4(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Lean_Elab_OpenDecl_resolveNameUsingNamespaces___at_Lean_Elab_Command_elabExport___spec__5(x_1, x_2, x_3, x_4, x_5); lean_dec(x_4); lean_dec(x_2); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Elab_addConstInfo___at_Lean_Elab_Command_elabExport___spec__22___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__26___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_elabExport___spec__26(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at_Lean_Elab_Command_elabExport___spec__25___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_getConstInfo___at_Lean_Elab_Command_elabExport___spec__25(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_mkConstWithLevelParams___at_Lean_Elab_Command_elabExport___spec__24___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_mkConstWithLevelParams___at_Lean_Elab_Command_elabExport___spec__24(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_addConstInfo___at_Lean_Elab_Command_elabExport___spec__23___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; -x_7 = l_Lean_Elab_addConstInfo___at_Lean_Elab_Command_elabExport___spec__22(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Lean_Elab_addConstInfo___at_Lean_Elab_Command_elabExport___spec__23(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_forInUnsafe_loop___at_Lean_Elab_Command_elabExport___spec__23___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabExport___spec__27___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; -x_9 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabExport___spec__23___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabExport___spec__27___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); return x_9; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabExport___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabExport___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_object* x_8, lean_object* x_9) { _start: { size_t x_10; size_t x_11; lean_object* x_12; @@ -9528,13 +9918,13 @@ x_10 = lean_unbox_usize(x_4); lean_dec(x_4); x_11 = lean_unbox_usize(x_5); lean_dec(x_5); -x_12 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabExport___spec__23(x_1, x_2, x_3, x_10, x_11, x_6, x_7, x_8, x_9); +x_12 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabExport___spec__27(x_1, x_2, x_3, x_10, x_11, x_6, x_7, x_8, x_9); lean_dec(x_8); lean_dec(x_3); return x_12; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabExport___spec__24___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabExport___spec__28___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; @@ -9542,7 +9932,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_Command_elabExport___spec__24(x_1, x_5, x_6, x_4); +x_7 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabExport___spec__28(x_1, x_5, x_6, x_4); lean_dec(x_1); return x_7; } @@ -9997,12 +10387,12 @@ uint8_t x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_obje lean_dec(x_20); lean_free_object(x_15); x_22 = 1; -x_23 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__1; +x_23 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__1; x_24 = l_Lean_Name_toString(x_1, x_22, x_23); -x_25 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__2; +x_25 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__2; x_26 = lean_string_append(x_25, x_24); lean_dec(x_24); -x_27 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__3; +x_27 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__3; x_28 = lean_string_append(x_26, x_27); x_29 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_29, 0, x_28); @@ -10067,12 +10457,12 @@ else 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; lean_object* x_55; lean_dec(x_39); x_42 = 1; -x_43 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__1; +x_43 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__1; x_44 = l_Lean_Name_toString(x_1, x_42, x_43); -x_45 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__2; +x_45 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__2; x_46 = lean_string_append(x_45, x_44); lean_dec(x_44); -x_47 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__3; +x_47 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__3; x_48 = lean_string_append(x_46, x_47); x_49 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_49, 0, x_48); @@ -10322,7 +10712,7 @@ lean_dec(x_6); x_9 = l_Lean_Syntax_getId(x_1); lean_dec(x_1); x_10 = 1; -x_11 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__1; +x_11 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__1; x_12 = l_Lean_Name_toString(x_9, x_10, x_11); x_13 = l_Lean_resolveUniqueNamespace___at_Lean_Elab_Command_elabOpen___spec__3___closed__1; x_14 = lean_string_append(x_13, x_12); @@ -10332,7 +10722,7 @@ x_16 = lean_string_append(x_14, x_15); x_17 = l_List_toString___at_Lean_OpenDecl_instToString___spec__1(x_7); x_18 = lean_string_append(x_16, x_17); lean_dec(x_17); -x_19 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__3; +x_19 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__3; x_20 = lean_string_append(x_18, x_19); x_21 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_21, 0, x_20); @@ -10388,7 +10778,7 @@ lean_dec(x_6); x_32 = l_Lean_Syntax_getId(x_1); lean_dec(x_1); x_33 = 1; -x_34 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__1; +x_34 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__1; x_35 = l_Lean_Name_toString(x_32, x_33, x_34); x_36 = l_Lean_resolveUniqueNamespace___at_Lean_Elab_Command_elabOpen___spec__3___closed__1; x_37 = lean_string_append(x_36, x_35); @@ -10398,7 +10788,7 @@ x_39 = lean_string_append(x_37, x_38); x_40 = l_List_toString___at_Lean_OpenDecl_instToString___spec__1(x_7); x_41 = lean_string_append(x_39, x_40); lean_dec(x_40); -x_42 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__3; +x_42 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__3; x_43 = lean_string_append(x_41, x_42); x_44 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_44, 0, x_43); @@ -10664,11 +11054,11 @@ lean_free_object(x_6); x_12 = lean_box(0); x_13 = l_Lean_Expr_const___override(x_1, x_12); x_14 = l_Lean_MessageData_ofExpr(x_13); -x_15 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__11___closed__2; +x_15 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__12___closed__2; x_16 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_16, 0, x_15); lean_ctor_set(x_16, 1, x_14); -x_17 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__11___closed__3; +x_17 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__12___closed__3; x_18 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_18, 0, x_16); lean_ctor_set(x_18, 1, x_17); @@ -10705,11 +11095,11 @@ lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean x_25 = lean_box(0); x_26 = l_Lean_Expr_const___override(x_1, x_25); x_27 = l_Lean_MessageData_ofExpr(x_26); -x_28 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__11___closed__2; +x_28 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__12___closed__2; x_29 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_29, 0, x_28); lean_ctor_set(x_29, 1, x_27); -x_30 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__11___closed__3; +x_30 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__12___closed__3; x_31 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_31, 0, x_29); lean_ctor_set(x_31, 1, x_30); @@ -11213,7 +11603,7 @@ lean_inc(x_21); lean_dec(x_12); lean_inc(x_7); lean_inc(x_1); -x_22 = l_Lean_Elab_OpenDecl_resolveId___at_Lean_Elab_Command_elabExport___spec__6(x_1, x_20, x_6, x_7, x_8, x_9); +x_22 = l_Lean_Elab_OpenDecl_resolveId___at_Lean_Elab_Command_elabExport___spec__7(x_1, x_20, x_6, x_7, x_8, x_9); if (lean_obj_tag(x_22) == 0) { lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; @@ -11535,7 +11925,7 @@ lean_dec(x_5); x_12 = lean_array_uget(x_2, x_4); lean_inc(x_7); lean_inc(x_1); -x_13 = l_Lean_Elab_OpenDecl_resolveId___at_Lean_Elab_Command_elabExport___spec__6(x_1, x_12, x_6, x_7, x_8, x_9); +x_13 = l_Lean_Elab_OpenDecl_resolveId___at_Lean_Elab_Command_elabExport___spec__7(x_1, x_12, x_6, x_7, x_8, 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; lean_object* x_18; uint8_t x_19; @@ -11666,7 +12056,7 @@ lean_dec(x_5); x_12 = lean_array_uget(x_2, x_4); lean_inc(x_7); lean_inc(x_1); -x_13 = l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5(x_1, x_12, x_6, x_7, x_8, x_9); +x_13 = l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6(x_1, x_12, x_6, x_7, x_8, 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; lean_object* x_18; uint8_t x_19; @@ -15446,16 +15836,104 @@ x_4 = lean_box(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__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_object* x_9; uint8_t x_10; -x_6 = l_Lean_Elab_Command_getRef(x_3, x_4, x_5); -x_7 = lean_ctor_get(x_6, 0); -lean_inc(x_7); -x_8 = lean_ctor_get(x_6, 1); -lean_inc(x_8); -lean_dec(x_6); +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_5 = l_Lean_Elab_Command_getRef(x_2, x_3, x_4); +x_6 = lean_ctor_get(x_5, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_5, 1); +lean_inc(x_7); +lean_dec(x_5); +x_8 = lean_ctor_get(x_2, 4); +lean_inc(x_8); +lean_inc(x_8); +x_9 = l_Lean_Elab_getBetterRef(x_6, x_8); +lean_dec(x_6); +x_10 = l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1(x_1, x_2, x_3, x_7); +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_12 = lean_ctor_get(x_10, 0); +x_13 = lean_ctor_get(x_10, 1); +x_14 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_12, x_8, x_2, x_3, x_13); +lean_dec(x_2); +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 0) +{ +lean_object* x_16; +x_16 = lean_ctor_get(x_14, 0); +lean_ctor_set(x_10, 1, x_16); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set_tag(x_14, 1); +lean_ctor_set(x_14, 0, x_10); +return x_14; +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_14, 0); +x_18 = lean_ctor_get(x_14, 1); +lean_inc(x_18); +lean_inc(x_17); +lean_dec(x_14); +lean_ctor_set(x_10, 1, x_17); +lean_ctor_set(x_10, 0, x_9); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_10); +lean_ctor_set(x_19, 1, 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; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_20 = lean_ctor_get(x_10, 0); +x_21 = lean_ctor_get(x_10, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_10); +x_22 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_20, x_8, x_2, x_3, x_21); +lean_dec(x_2); +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +if (lean_is_exclusive(x_22)) { + lean_ctor_release(x_22, 0); + lean_ctor_release(x_22, 1); + x_25 = x_22; +} else { + lean_dec_ref(x_22); + x_25 = lean_box(0); +} +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_9); +lean_ctor_set(x_26, 1, x_23); +if (lean_is_scalar(x_25)) { + x_27 = lean_alloc_ctor(1, 2, 0); +} else { + x_27 = x_25; + lean_ctor_set_tag(x_27, 1); +} +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_24); +return x_27; +} +} +} +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; +x_6 = l_Lean_Elab_Command_getRef(x_3, x_4, x_5); +x_7 = lean_ctor_get(x_6, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_6, 1); +lean_inc(x_8); +lean_dec(x_6); x_9 = l_Lean_replaceRef(x_1, x_7); lean_dec(x_7); x_10 = !lean_is_exclusive(x_3); @@ -15465,7 +15943,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_expandDeclId___spec__18(x_2, x_3, x_4, x_8); +x_12 = l_Lean_throwError___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__2(x_2, x_3, x_4, x_8); return x_12; } else @@ -15503,12 +15981,12 @@ lean_ctor_set(x_23, 7, x_19); lean_ctor_set(x_23, 8, x_20); lean_ctor_set(x_23, 9, x_21); lean_ctor_set_uint8(x_23, sizeof(void*)*10, x_22); -x_24 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__18(x_2, x_23, x_4, x_8); +x_24 = l_Lean_throwError___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__2(x_2, x_23, x_4, x_8); return x_24; } } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__2___closed__1() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__3___closed__1() { _start: { lean_object* x_1; @@ -15516,16 +15994,16 @@ x_1 = lean_mk_string_unchecked("redundant binder annotation update", 34, 34); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__2___closed__2() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__3___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__2___closed__1; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__3___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___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) { _start: { uint8_t x_9; @@ -15559,7 +16037,7 @@ goto _start; else { lean_object* x_17; lean_object* x_18; uint8_t x_19; -x_17 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__2___closed__2; +x_17 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__3___closed__2; x_18 = l_Lean_throwErrorAt___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__1(x_11, x_17, x_6, x_7, x_8); lean_dec(x_11); x_19 = !lean_is_exclusive(x_18); @@ -15584,7 +16062,7 @@ return x_22; } } } -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__3(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_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4) { _start: { uint8_t x_5; @@ -15618,7 +16096,7 @@ return x_12; } } } -LEAN_EXPORT uint8_t l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___lambda__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___lambda__1(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; @@ -15641,7 +16119,7 @@ return x_7; } } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__1() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__1() { _start: { lean_object* x_1; @@ -15649,7 +16127,7 @@ x_1 = lean_mk_string_unchecked("{", 1, 1); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__2() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__2() { _start: { lean_object* x_1; @@ -15657,17 +16135,17 @@ x_1 = lean_mk_string_unchecked("null", 4, 4); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__3() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__3() { _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_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__2; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__2; 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_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__4() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__4() { _start: { lean_object* x_1; @@ -15675,7 +16153,7 @@ x_1 = lean_mk_string_unchecked("}", 1, 1); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__5() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__5() { _start: { lean_object* x_1; lean_object* x_2; @@ -15684,7 +16162,7 @@ x_2 = l_Array_append___rarg(x_1, x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__6() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__6() { _start: { lean_object* x_1; @@ -15692,7 +16170,7 @@ x_1 = lean_mk_string_unchecked("(", 1, 1); return x_1; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4(uint8_t x_1, lean_object* 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_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5(uint8_t x_1, lean_object* 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) { _start: { uint8_t x_11; @@ -15735,7 +16213,7 @@ if (lean_is_exclusive(x_21)) { x_26 = lean_box(0); } lean_inc(x_13); -x_295 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___lambda__1___boxed), 2, 1); +x_295 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___lambda__1___boxed), 2, 1); lean_closure_set(x_295, 0, x_13); x_296 = lean_unsigned_to_nat(0u); x_297 = l_Array_findIdx_x3f_loop___rarg(x_22, x_295, x_296); @@ -15817,15 +16295,15 @@ lean_object* x_316; lean_object* x_317; lean_object* x_318; lean_object* x_319; x_316 = lean_ctor_get(x_314, 1); x_317 = lean_ctor_get(x_314, 0); lean_dec(x_317); -x_318 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__1; +x_318 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__1; lean_inc(x_309); lean_ctor_set_tag(x_314, 2); lean_ctor_set(x_314, 1, x_318); lean_ctor_set(x_314, 0, x_309); -x_319 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__3; +x_319 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__3; lean_inc(x_309); x_320 = l_Lean_Syntax_node1(x_309, x_319, x_13); -x_321 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__4; +x_321 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__4; lean_inc(x_309); lean_ctor_set_tag(x_310, 2); lean_ctor_set(x_310, 1, x_321); @@ -15833,7 +16311,7 @@ lean_ctor_set(x_310, 0, x_309); if (lean_obj_tag(x_2) == 0) { lean_object* x_322; lean_object* x_323; lean_object* x_324; lean_object* x_325; lean_object* x_326; uint8_t x_327; lean_object* x_328; lean_object* x_329; lean_object* x_330; -x_322 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__5; +x_322 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__5; lean_inc(x_309); x_323 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_323, 0, x_309); @@ -15864,7 +16342,7 @@ else lean_object* x_331; lean_object* x_332; lean_object* x_333; lean_object* x_334; lean_object* x_335; lean_object* x_336; lean_object* x_337; lean_object* x_338; lean_object* x_339; uint8_t x_340; lean_object* x_341; lean_object* x_342; lean_object* x_343; lean_object* x_344; x_331 = lean_ctor_get(x_2, 0); lean_inc(x_331); -x_332 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__1; +x_332 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__1; lean_inc(x_309); lean_ctor_set_tag(x_304, 2); lean_ctor_set(x_304, 1, x_332); @@ -15906,15 +16384,15 @@ lean_object* x_345; lean_object* x_346; lean_object* x_347; lean_object* x_348; x_345 = lean_ctor_get(x_314, 1); lean_inc(x_345); lean_dec(x_314); -x_346 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__1; +x_346 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__1; lean_inc(x_309); x_347 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_347, 0, x_309); lean_ctor_set(x_347, 1, x_346); -x_348 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__3; +x_348 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__3; lean_inc(x_309); x_349 = l_Lean_Syntax_node1(x_309, x_348, x_13); -x_350 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__4; +x_350 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__4; lean_inc(x_309); lean_ctor_set_tag(x_310, 2); lean_ctor_set(x_310, 1, x_350); @@ -15922,7 +16400,7 @@ lean_ctor_set(x_310, 0, x_309); if (lean_obj_tag(x_2) == 0) { lean_object* x_351; lean_object* x_352; lean_object* x_353; lean_object* x_354; lean_object* x_355; uint8_t x_356; lean_object* x_357; lean_object* x_358; lean_object* x_359; -x_351 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__5; +x_351 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__5; lean_inc(x_309); x_352 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_352, 0, x_309); @@ -15953,7 +16431,7 @@ else 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; uint8_t x_369; lean_object* x_370; lean_object* x_371; lean_object* x_372; lean_object* x_373; x_360 = lean_ctor_get(x_2, 0); lean_inc(x_360); -x_361 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__1; +x_361 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__1; lean_inc(x_309); lean_ctor_set_tag(x_304, 2); lean_ctor_set(x_304, 1, x_361); @@ -16007,7 +16485,7 @@ if (lean_is_exclusive(x_375)) { lean_dec_ref(x_375); x_377 = lean_box(0); } -x_378 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__1; +x_378 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__1; lean_inc(x_309); if (lean_is_scalar(x_377)) { x_379 = lean_alloc_ctor(2, 2, 0); @@ -16017,10 +16495,10 @@ if (lean_is_scalar(x_377)) { } lean_ctor_set(x_379, 0, x_309); lean_ctor_set(x_379, 1, x_378); -x_380 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__3; +x_380 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__3; lean_inc(x_309); x_381 = l_Lean_Syntax_node1(x_309, x_380, x_13); -x_382 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__4; +x_382 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__4; lean_inc(x_309); x_383 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_383, 0, x_309); @@ -16028,7 +16506,7 @@ lean_ctor_set(x_383, 1, x_382); if (lean_obj_tag(x_2) == 0) { lean_object* x_384; lean_object* x_385; lean_object* x_386; lean_object* x_387; lean_object* x_388; uint8_t x_389; lean_object* x_390; lean_object* x_391; lean_object* x_392; -x_384 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__5; +x_384 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__5; lean_inc(x_309); x_385 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_385, 0, x_309); @@ -16059,7 +16537,7 @@ else lean_object* x_393; lean_object* x_394; lean_object* x_395; lean_object* x_396; lean_object* x_397; lean_object* x_398; lean_object* x_399; lean_object* x_400; lean_object* x_401; uint8_t x_402; lean_object* x_403; lean_object* x_404; lean_object* x_405; lean_object* x_406; x_393 = lean_ctor_get(x_2, 0); lean_inc(x_393); -x_394 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__1; +x_394 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__1; lean_inc(x_309); lean_ctor_set_tag(x_304, 2); lean_ctor_set(x_304, 1, x_394); @@ -16129,7 +16607,7 @@ if (lean_is_exclusive(x_414)) { lean_dec_ref(x_414); x_416 = lean_box(0); } -x_417 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__1; +x_417 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__1; lean_inc(x_410); if (lean_is_scalar(x_416)) { x_418 = lean_alloc_ctor(2, 2, 0); @@ -16139,10 +16617,10 @@ if (lean_is_scalar(x_416)) { } lean_ctor_set(x_418, 0, x_410); lean_ctor_set(x_418, 1, x_417); -x_419 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__3; +x_419 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__3; lean_inc(x_410); x_420 = l_Lean_Syntax_node1(x_410, x_419, x_13); -x_421 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__4; +x_421 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__4; lean_inc(x_410); if (lean_is_scalar(x_413)) { x_422 = lean_alloc_ctor(2, 2, 0); @@ -16155,7 +16633,7 @@ lean_ctor_set(x_422, 1, x_421); if (lean_obj_tag(x_2) == 0) { lean_object* x_423; lean_object* x_424; lean_object* x_425; lean_object* x_426; lean_object* x_427; uint8_t x_428; lean_object* x_429; lean_object* x_430; lean_object* x_431; lean_object* x_432; -x_423 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__5; +x_423 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__5; lean_inc(x_410); x_424 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_424, 0, x_410); @@ -16187,7 +16665,7 @@ else lean_object* x_433; lean_object* x_434; lean_object* x_435; lean_object* x_436; lean_object* x_437; lean_object* x_438; lean_object* x_439; lean_object* x_440; lean_object* x_441; lean_object* x_442; uint8_t x_443; lean_object* x_444; lean_object* x_445; lean_object* x_446; lean_object* x_447; x_433 = lean_ctor_get(x_2, 0); lean_inc(x_433); -x_434 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__1; +x_434 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__1; lean_inc(x_410); x_435 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_435, 0, x_410); @@ -16253,12 +16731,12 @@ lean_object* x_460; lean_object* x_461; lean_object* x_462; lean_object* x_463; x_460 = lean_ctor_get(x_458, 1); x_461 = lean_ctor_get(x_458, 0); lean_dec(x_461); -x_462 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__6; +x_462 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__6; lean_inc(x_453); lean_ctor_set_tag(x_458, 2); lean_ctor_set(x_458, 1, x_462); lean_ctor_set(x_458, 0, x_453); -x_463 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__3; +x_463 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__3; lean_inc(x_453); x_464 = l_Lean_Syntax_node1(x_453, x_463, x_13); x_465 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___closed__12; @@ -16275,7 +16753,7 @@ lean_ctor_set(x_454, 0, x_453); if (lean_obj_tag(x_2) == 0) { lean_object* x_468; lean_object* x_469; lean_object* x_470; lean_object* x_471; lean_object* x_472; uint8_t x_473; lean_object* x_474; lean_object* x_475; lean_object* x_476; -x_468 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__5; +x_468 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__5; lean_inc(x_453); x_469 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_469, 0, x_453); @@ -16306,7 +16784,7 @@ else 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; uint8_t x_485; lean_object* x_486; lean_object* x_487; lean_object* x_488; lean_object* x_489; x_477 = lean_ctor_get(x_2, 0); lean_inc(x_477); -x_478 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__1; +x_478 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__1; lean_inc(x_453); lean_ctor_set_tag(x_448, 2); lean_ctor_set(x_448, 1, x_478); @@ -16347,12 +16825,12 @@ lean_object* x_490; lean_object* x_491; lean_object* x_492; lean_object* x_493; x_490 = lean_ctor_get(x_458, 1); lean_inc(x_490); lean_dec(x_458); -x_491 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__6; +x_491 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__6; lean_inc(x_453); x_492 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_492, 0, x_453); lean_ctor_set(x_492, 1, x_491); -x_493 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__3; +x_493 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__3; lean_inc(x_453); x_494 = l_Lean_Syntax_node1(x_453, x_493, x_13); x_495 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___closed__12; @@ -16369,7 +16847,7 @@ lean_ctor_set(x_454, 0, x_453); if (lean_obj_tag(x_2) == 0) { lean_object* x_498; lean_object* x_499; lean_object* x_500; lean_object* x_501; lean_object* x_502; uint8_t x_503; lean_object* x_504; lean_object* x_505; lean_object* x_506; -x_498 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__5; +x_498 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__5; lean_inc(x_453); x_499 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_499, 0, x_453); @@ -16400,7 +16878,7 @@ else 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; uint8_t x_515; lean_object* x_516; lean_object* x_517; lean_object* x_518; lean_object* x_519; x_507 = lean_ctor_get(x_2, 0); lean_inc(x_507); -x_508 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__1; +x_508 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__1; lean_inc(x_453); lean_ctor_set_tag(x_448, 2); lean_ctor_set(x_448, 1, x_508); @@ -16453,7 +16931,7 @@ if (lean_is_exclusive(x_521)) { lean_dec_ref(x_521); x_523 = lean_box(0); } -x_524 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__6; +x_524 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__6; lean_inc(x_453); if (lean_is_scalar(x_523)) { x_525 = lean_alloc_ctor(2, 2, 0); @@ -16463,7 +16941,7 @@ if (lean_is_scalar(x_523)) { } lean_ctor_set(x_525, 0, x_453); lean_ctor_set(x_525, 1, x_524); -x_526 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__3; +x_526 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__3; lean_inc(x_453); x_527 = l_Lean_Syntax_node1(x_453, x_526, x_13); x_528 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___closed__12; @@ -16480,7 +16958,7 @@ lean_ctor_set(x_531, 1, x_530); if (lean_obj_tag(x_2) == 0) { 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; lean_object* x_539; lean_object* x_540; -x_532 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__5; +x_532 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__5; lean_inc(x_453); x_533 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_533, 0, x_453); @@ -16511,7 +16989,7 @@ else 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; uint8_t x_549; lean_object* x_550; lean_object* x_551; lean_object* x_552; lean_object* x_553; x_541 = lean_ctor_get(x_2, 0); lean_inc(x_541); -x_542 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__1; +x_542 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__1; lean_inc(x_453); lean_ctor_set_tag(x_448, 2); lean_ctor_set(x_448, 1, x_542); @@ -16580,7 +17058,7 @@ if (lean_is_exclusive(x_561)) { lean_dec_ref(x_561); x_563 = lean_box(0); } -x_564 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__6; +x_564 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__6; lean_inc(x_557); if (lean_is_scalar(x_563)) { x_565 = lean_alloc_ctor(2, 2, 0); @@ -16590,7 +17068,7 @@ if (lean_is_scalar(x_563)) { } lean_ctor_set(x_565, 0, x_557); lean_ctor_set(x_565, 1, x_564); -x_566 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__3; +x_566 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__3; lean_inc(x_557); x_567 = l_Lean_Syntax_node1(x_557, x_566, x_13); x_568 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___closed__12; @@ -16612,7 +17090,7 @@ lean_ctor_set(x_571, 1, x_570); if (lean_obj_tag(x_2) == 0) { lean_object* x_572; lean_object* x_573; lean_object* x_574; lean_object* x_575; lean_object* x_576; uint8_t x_577; lean_object* x_578; lean_object* x_579; lean_object* x_580; lean_object* x_581; -x_572 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__5; +x_572 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__5; lean_inc(x_557); x_573 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_573, 0, x_557); @@ -16644,7 +17122,7 @@ else 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; uint8_t x_591; lean_object* x_592; lean_object* x_593; lean_object* x_594; lean_object* x_595; x_582 = lean_ctor_get(x_2, 0); lean_inc(x_582); -x_583 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__1; +x_583 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__1; lean_inc(x_557); x_584 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_584, 0, x_557); @@ -16726,15 +17204,15 @@ lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean x_40 = lean_ctor_get(x_38, 1); x_41 = lean_ctor_get(x_38, 0); lean_dec(x_41); -x_42 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__1; +x_42 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__1; lean_inc(x_33); lean_ctor_set_tag(x_38, 2); lean_ctor_set(x_38, 1, x_42); lean_ctor_set(x_38, 0, x_33); -x_43 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__3; +x_43 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__3; lean_inc(x_33); x_44 = l_Lean_Syntax_node1(x_33, x_43, x_13); -x_45 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__4; +x_45 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__4; lean_inc(x_33); lean_ctor_set_tag(x_34, 2); lean_ctor_set(x_34, 1, x_45); @@ -16743,7 +17221,7 @@ if (lean_obj_tag(x_2) == 0) { lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_free_object(x_28); -x_46 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__5; +x_46 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__5; lean_inc(x_33); x_47 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_47, 0, x_33); @@ -16777,7 +17255,7 @@ else lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; 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_54 = lean_ctor_get(x_2, 0); lean_inc(x_54); -x_55 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__1; +x_55 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__1; lean_inc(x_33); lean_ctor_set_tag(x_28, 2); lean_ctor_set(x_28, 1, x_55); @@ -16821,15 +17299,15 @@ lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean x_66 = lean_ctor_get(x_38, 1); lean_inc(x_66); lean_dec(x_38); -x_67 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__1; +x_67 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__1; lean_inc(x_33); x_68 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_68, 0, x_33); lean_ctor_set(x_68, 1, x_67); -x_69 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__3; +x_69 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__3; lean_inc(x_33); x_70 = l_Lean_Syntax_node1(x_33, x_69, x_13); -x_71 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__4; +x_71 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__4; lean_inc(x_33); lean_ctor_set_tag(x_34, 2); lean_ctor_set(x_34, 1, x_71); @@ -16838,7 +17316,7 @@ if (lean_obj_tag(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_free_object(x_28); -x_72 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__5; +x_72 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__5; lean_inc(x_33); x_73 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_73, 0, x_33); @@ -16872,7 +17350,7 @@ else lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; x_80 = lean_ctor_get(x_2, 0); lean_inc(x_80); -x_81 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__1; +x_81 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__1; lean_inc(x_33); lean_ctor_set_tag(x_28, 2); lean_ctor_set(x_28, 1, x_81); @@ -16928,7 +17406,7 @@ if (lean_is_exclusive(x_93)) { lean_dec_ref(x_93); x_95 = lean_box(0); } -x_96 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__1; +x_96 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__1; lean_inc(x_33); if (lean_is_scalar(x_95)) { x_97 = lean_alloc_ctor(2, 2, 0); @@ -16938,10 +17416,10 @@ if (lean_is_scalar(x_95)) { } lean_ctor_set(x_97, 0, x_33); lean_ctor_set(x_97, 1, x_96); -x_98 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__3; +x_98 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__3; lean_inc(x_33); x_99 = l_Lean_Syntax_node1(x_33, x_98, x_13); -x_100 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__4; +x_100 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__4; lean_inc(x_33); x_101 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_101, 0, x_33); @@ -16950,7 +17428,7 @@ if (lean_obj_tag(x_2) == 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_free_object(x_28); -x_102 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__5; +x_102 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__5; lean_inc(x_33); x_103 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_103, 0, x_33); @@ -16984,7 +17462,7 @@ else lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; x_110 = lean_ctor_get(x_2, 0); lean_inc(x_110); -x_111 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__1; +x_111 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__1; lean_inc(x_33); lean_ctor_set_tag(x_28, 2); lean_ctor_set(x_28, 1, x_111); @@ -17056,7 +17534,7 @@ if (lean_is_exclusive(x_129)) { lean_dec_ref(x_129); x_131 = lean_box(0); } -x_132 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__1; +x_132 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__1; lean_inc(x_125); if (lean_is_scalar(x_131)) { x_133 = lean_alloc_ctor(2, 2, 0); @@ -17066,10 +17544,10 @@ if (lean_is_scalar(x_131)) { } lean_ctor_set(x_133, 0, x_125); lean_ctor_set(x_133, 1, x_132); -x_134 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__3; +x_134 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__3; lean_inc(x_125); x_135 = l_Lean_Syntax_node1(x_125, x_134, x_13); -x_136 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__4; +x_136 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__4; lean_inc(x_125); if (lean_is_scalar(x_128)) { x_137 = lean_alloc_ctor(2, 2, 0); @@ -17082,7 +17560,7 @@ lean_ctor_set(x_137, 1, x_136); if (lean_obj_tag(x_2) == 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; -x_138 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__5; +x_138 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__5; lean_inc(x_125); x_139 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_139, 0, x_125); @@ -17116,7 +17594,7 @@ 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; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; x_146 = lean_ctor_get(x_2, 0); lean_inc(x_146); -x_147 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__1; +x_147 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__1; lean_inc(x_125); x_148 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_148, 0, x_125); @@ -17184,12 +17662,12 @@ lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; x_171 = lean_ctor_get(x_169, 1); x_172 = lean_ctor_get(x_169, 0); lean_dec(x_172); -x_173 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__6; +x_173 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__6; lean_inc(x_164); lean_ctor_set_tag(x_169, 2); lean_ctor_set(x_169, 1, x_173); lean_ctor_set(x_169, 0, x_164); -x_174 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__3; +x_174 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__3; lean_inc(x_164); x_175 = l_Lean_Syntax_node1(x_164, x_174, x_13); x_176 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___closed__12; @@ -17207,7 +17685,7 @@ if (lean_obj_tag(x_2) == 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_free_object(x_159); -x_179 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__5; +x_179 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__5; lean_inc(x_164); x_180 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_180, 0, x_164); @@ -17241,7 +17719,7 @@ else 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_187 = lean_ctor_get(x_2, 0); lean_inc(x_187); -x_188 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__1; +x_188 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__1; lean_inc(x_164); lean_ctor_set_tag(x_159, 2); lean_ctor_set(x_159, 1, x_188); @@ -17284,12 +17762,12 @@ lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; x_198 = lean_ctor_get(x_169, 1); lean_inc(x_198); lean_dec(x_169); -x_199 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__6; +x_199 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__6; lean_inc(x_164); x_200 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_200, 0, x_164); lean_ctor_set(x_200, 1, x_199); -x_201 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__3; +x_201 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__3; lean_inc(x_164); x_202 = l_Lean_Syntax_node1(x_164, x_201, x_13); x_203 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___closed__12; @@ -17307,7 +17785,7 @@ if (lean_obj_tag(x_2) == 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_free_object(x_159); -x_206 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__5; +x_206 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__5; lean_inc(x_164); x_207 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_207, 0, x_164); @@ -17341,7 +17819,7 @@ else 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_214 = lean_ctor_get(x_2, 0); lean_inc(x_214); -x_215 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__1; +x_215 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__1; lean_inc(x_164); lean_ctor_set_tag(x_159, 2); lean_ctor_set(x_159, 1, x_215); @@ -17396,7 +17874,7 @@ if (lean_is_exclusive(x_226)) { lean_dec_ref(x_226); x_228 = lean_box(0); } -x_229 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__6; +x_229 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__6; lean_inc(x_164); if (lean_is_scalar(x_228)) { x_230 = lean_alloc_ctor(2, 2, 0); @@ -17406,7 +17884,7 @@ if (lean_is_scalar(x_228)) { } lean_ctor_set(x_230, 0, x_164); lean_ctor_set(x_230, 1, x_229); -x_231 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__3; +x_231 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__3; lean_inc(x_164); x_232 = l_Lean_Syntax_node1(x_164, x_231, x_13); x_233 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___closed__12; @@ -17424,7 +17902,7 @@ if (lean_obj_tag(x_2) == 0) { lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_free_object(x_159); -x_237 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__5; +x_237 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__5; lean_inc(x_164); x_238 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_238, 0, x_164); @@ -17458,7 +17936,7 @@ else lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; x_245 = lean_ctor_get(x_2, 0); lean_inc(x_245); -x_246 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__1; +x_246 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__1; lean_inc(x_164); lean_ctor_set_tag(x_159, 2); lean_ctor_set(x_159, 1, x_246); @@ -17529,7 +18007,7 @@ if (lean_is_exclusive(x_263)) { lean_dec_ref(x_263); x_265 = lean_box(0); } -x_266 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__6; +x_266 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__6; lean_inc(x_259); if (lean_is_scalar(x_265)) { x_267 = lean_alloc_ctor(2, 2, 0); @@ -17539,7 +18017,7 @@ if (lean_is_scalar(x_265)) { } lean_ctor_set(x_267, 0, x_259); lean_ctor_set(x_267, 1, x_266); -x_268 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__3; +x_268 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__3; lean_inc(x_259); x_269 = l_Lean_Syntax_node1(x_259, x_268, x_13); x_270 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___closed__12; @@ -17561,7 +18039,7 @@ lean_ctor_set(x_273, 1, x_272); if (lean_obj_tag(x_2) == 0) { lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; -x_274 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__5; +x_274 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__5; lean_inc(x_259); x_275 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_275, 0, x_259); @@ -17595,7 +18073,7 @@ else 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; x_282 = lean_ctor_get(x_2, 0); lean_inc(x_282); -x_283 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__1; +x_283 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__1; lean_inc(x_259); x_284 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_284, 0, x_259); @@ -17637,7 +18115,7 @@ goto block_20; } } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__1() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6___closed__1() { _start: { lean_object* x_1; @@ -17645,16 +18123,16 @@ x_1 = lean_mk_string_unchecked("cannot change the binder annotation of the previ return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__2() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__1; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__3() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6___closed__3() { _start: { lean_object* x_1; @@ -17662,16 +18140,16 @@ x_1 = lean_mk_string_unchecked("`", 1, 1); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__4() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__3; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6___closed__3; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5(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_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___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) { _start: { uint8_t x_10; @@ -17725,11 +18203,11 @@ else { lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; x_25 = l_Lean_MessageData_ofName(x_19); -x_26 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__2; +x_26 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6___closed__2; x_27 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_27, 0, x_26); lean_ctor_set(x_27, 1, x_25); -x_28 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__4; +x_28 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6___closed__4; x_29 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_29, 0, x_27); lean_ctor_set(x_29, 1, x_28); @@ -17758,7 +18236,7 @@ return x_34; } } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6___closed__1() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___closed__1() { _start: { lean_object* x_1; @@ -17766,16 +18244,16 @@ x_1 = lean_mk_string_unchecked("cannot update binder annotation of variables wit return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6___closed__2() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6___closed__1; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7(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) { _start: { uint8_t x_9; @@ -17809,7 +18287,7 @@ goto _start; else { lean_object* x_17; lean_object* x_18; uint8_t x_19; -x_17 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6___closed__2; +x_17 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___closed__2; x_18 = l_Lean_throwErrorAt___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__1(x_11, x_17, x_6, x_7, x_8); lean_dec(x_11); x_19 = !lean_is_exclusive(x_18); @@ -17834,7 +18312,7 @@ return x_22; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___lambda__1(lean_object* x_1, uint8_t 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_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___lambda__1(lean_object* x_1, uint8_t x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { lean_object* x_10; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; @@ -17934,7 +18412,7 @@ lean_dec(x_21); x_22 = lean_array_size(x_3); x_23 = 0; x_24 = lean_box(0); -x_25 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__2(x_18, x_3, x_22, x_23, x_24, x_7, x_8, x_9); +x_25 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__3(x_18, x_3, x_22, x_23, x_24, x_7, x_8, x_9); lean_dec(x_18); if (lean_obj_tag(x_25) == 0) { @@ -18041,7 +18519,7 @@ size_t x_53; size_t x_54; uint8_t x_55; x_53 = 0; x_54 = lean_usize_of_nat(x_49); lean_dec(x_49); -x_55 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__3(x_18, x_3, x_53, x_54); +x_55 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4(x_18, x_3, x_53, x_54); if (x_55 == 0) { lean_object* x_56; @@ -18073,7 +18551,7 @@ lean_ctor_set(x_60, 1, x_59); x_61 = lean_array_size(x_57); x_62 = lean_unbox(x_46); lean_dec(x_46); -x_63 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4(x_2, x_45, x_62, x_57, x_61, x_53, x_60, x_7, x_8, x_9); +x_63 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5(x_2, x_45, x_62, x_57, x_61, x_53, x_60, x_7, x_8, x_9); lean_dec(x_7); lean_dec(x_57); x_64 = lean_ctor_get(x_63, 0); @@ -18207,7 +18685,7 @@ return x_92; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___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_14; lean_object* x_15; lean_object* x_16; @@ -18224,7 +18702,7 @@ x_16 = lean_apply_7(x_2, x_3, x_4, x_5, x_15, x_8, x_9, x_10); return x_16; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { uint8_t x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; @@ -18240,7 +18718,7 @@ x_15 = lean_apply_7(x_3, x_4, x_5, x_6, x_14, x_8, x_9, x_10); return x_15; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___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; @@ -18253,7 +18731,7 @@ if (lean_obj_tag(x_14) == 0) { lean_object* x_16; lean_object* x_17; x_16 = lean_box(0); -x_17 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___lambda__3(x_8, x_15, x_3, x_4, x_5, x_6, x_16, x_9, x_10, x_11); +x_17 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___lambda__3(x_8, x_15, x_3, x_4, x_5, x_6, x_16, x_9, x_10, x_11); return x_17; } else @@ -18264,14 +18742,14 @@ x_18 = lean_array_size(x_4); x_19 = 0; x_20 = lean_box(0); lean_inc(x_9); -x_21 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6(x_15, x_4, x_18, x_19, x_20, x_9, x_10, x_11); +x_21 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7(x_15, x_4, x_18, x_19, x_20, x_9, x_10, x_11); 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 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___lambda__3(x_8, x_15, x_3, x_4, x_5, x_6, x_20, x_9, x_10, x_22); +x_23 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___lambda__3(x_8, x_15, x_3, x_4, x_5, x_6, x_20, x_9, x_10, x_22); return x_23; } else @@ -18307,7 +18785,7 @@ return x_27; } } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___closed__1() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___closed__1() { _start: { lean_object* x_1; @@ -18315,19 +18793,19 @@ x_1 = lean_mk_string_unchecked("instBinder", 10, 10); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___closed__2() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l___regBuiltin_Lean_Elab_Command_elabModuleDoc__1___closed__1; x_2 = l___regBuiltin_Lean_Elab_Command_elabModuleDoc__1___closed__2; x_3 = l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_typelessBinder_x3f___closed__1; -x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___closed__1; +x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___closed__1; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___closed__3() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -18339,7 +18817,7 @@ lean_ctor_set(x_3, 1, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7(uint8_t 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_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8(uint8_t 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) { _start: { uint8_t x_9; @@ -18372,7 +18850,7 @@ x_25 = lean_ctor_get(x_22, 0); x_26 = lean_ctor_get(x_22, 1); x_27 = lean_box(x_1); lean_inc(x_11); -x_28 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___lambda__1___boxed), 9, 2); +x_28 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___lambda__1___boxed), 9, 2); lean_closure_set(x_28, 0, x_11); lean_closure_set(x_28, 1, x_27); x_29 = l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_typelessBinder_x3f___closed__3; @@ -18388,7 +18866,7 @@ if (x_32 == 0) { lean_object* x_33; uint8_t x_34; lean_dec(x_28); -x_33 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___closed__2; +x_33 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___closed__2; lean_inc(x_11); x_34 = l_Lean_Syntax_isOfKind(x_11, x_33); if (x_34 == 0) @@ -18430,10 +18908,10 @@ x_44 = l_Lean_Syntax_getArg(x_38, x_43); lean_dec(x_38); x_45 = lean_array_size(x_24); x_46 = 0; -x_47 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___closed__3; +x_47 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___closed__3; x_48 = lean_box(0); lean_inc(x_6); -x_49 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5(x_47, x_44, x_24, x_45, x_46, x_48, x_6, x_7, x_8); +x_49 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6(x_47, x_44, x_24, x_45, x_46, x_48, x_6, x_7, x_8); lean_dec(x_44); if (lean_obj_tag(x_49) == 0) { @@ -18522,7 +19000,7 @@ lean_ctor_set(x_66, 0, x_65); x_67 = lean_box(0); lean_inc(x_7); lean_inc(x_6); -x_68 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___lambda__2(x_58, x_28, x_24, x_25, x_26, x_67, x_66, x_6, x_7, x_8); +x_68 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___lambda__2(x_58, x_28, x_24, x_25, x_26, x_67, x_66, x_6, x_7, x_8); lean_dec(x_58); if (lean_obj_tag(x_68) == 0) { @@ -18573,7 +19051,7 @@ x_75 = lean_box(0); x_76 = lean_box(0); lean_inc(x_7); lean_inc(x_6); -x_77 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___lambda__2(x_58, x_28, x_24, x_25, x_26, x_76, x_75, x_6, x_7, x_8); +x_77 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___lambda__2(x_58, x_28, x_24, x_25, x_26, x_76, x_75, x_6, x_7, x_8); lean_dec(x_58); if (lean_obj_tag(x_77) == 0) { @@ -18653,7 +19131,7 @@ lean_ctor_set(x_93, 0, x_92); x_94 = lean_box(0); lean_inc(x_7); lean_inc(x_6); -x_95 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___lambda__4(x_11, x_85, x_28, x_24, x_25, x_26, x_94, x_93, x_6, x_7, x_8); +x_95 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___lambda__4(x_11, x_85, x_28, x_24, x_25, x_26, x_94, x_93, x_6, x_7, x_8); lean_dec(x_85); lean_dec(x_11); if (lean_obj_tag(x_95) == 0) @@ -18704,7 +19182,7 @@ x_102 = lean_box(0); x_103 = lean_box(0); lean_inc(x_7); lean_inc(x_6); -x_104 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___lambda__4(x_11, x_85, x_28, x_24, x_25, x_26, x_103, x_102, x_6, x_7, x_8); +x_104 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___lambda__4(x_11, x_85, x_28, x_24, x_25, x_26, x_103, x_102, x_6, x_7, x_8); lean_dec(x_85); lean_dec(x_11); if (lean_obj_tag(x_104) == 0) @@ -18757,7 +19235,7 @@ lean_inc(x_112); lean_dec(x_22); x_114 = lean_box(x_1); lean_inc(x_11); -x_115 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___lambda__1___boxed), 9, 2); +x_115 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___lambda__1___boxed), 9, 2); lean_closure_set(x_115, 0, x_11); lean_closure_set(x_115, 1, x_114); x_116 = l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_typelessBinder_x3f___closed__3; @@ -18773,7 +19251,7 @@ if (x_119 == 0) { lean_object* x_120; uint8_t x_121; lean_dec(x_115); -x_120 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___closed__2; +x_120 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___closed__2; lean_inc(x_11); x_121 = l_Lean_Syntax_isOfKind(x_11, x_120); if (x_121 == 0) @@ -18821,10 +19299,10 @@ x_133 = l_Lean_Syntax_getArg(x_126, x_132); lean_dec(x_126); x_134 = lean_array_size(x_111); x_135 = 0; -x_136 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___closed__3; +x_136 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___closed__3; x_137 = lean_box(0); lean_inc(x_6); -x_138 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5(x_136, x_133, x_111, x_134, x_135, x_137, x_6, x_7, x_8); +x_138 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6(x_136, x_133, x_111, x_134, x_135, x_137, x_6, x_7, x_8); lean_dec(x_133); if (lean_obj_tag(x_138) == 0) { @@ -18919,7 +19397,7 @@ lean_ctor_set(x_157, 0, x_156); x_158 = lean_box(0); lean_inc(x_7); lean_inc(x_6); -x_159 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___lambda__2(x_148, x_115, x_111, x_112, x_113, x_158, x_157, x_6, x_7, x_8); +x_159 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___lambda__2(x_148, x_115, x_111, x_112, x_113, x_158, x_157, x_6, x_7, x_8); lean_dec(x_148); if (lean_obj_tag(x_159) == 0) { @@ -18971,7 +19449,7 @@ x_166 = lean_box(0); x_167 = lean_box(0); lean_inc(x_7); lean_inc(x_6); -x_168 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___lambda__2(x_148, x_115, x_111, x_112, x_113, x_167, x_166, x_6, x_7, x_8); +x_168 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___lambda__2(x_148, x_115, x_111, x_112, x_113, x_167, x_166, x_6, x_7, x_8); lean_dec(x_148); if (lean_obj_tag(x_168) == 0) { @@ -19055,7 +19533,7 @@ lean_ctor_set(x_185, 0, x_184); x_186 = lean_box(0); lean_inc(x_7); lean_inc(x_6); -x_187 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___lambda__4(x_11, x_176, x_115, x_111, x_112, x_113, x_186, x_185, x_6, x_7, x_8); +x_187 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___lambda__4(x_11, x_176, x_115, x_111, x_112, x_113, x_186, x_185, x_6, x_7, x_8); lean_dec(x_176); lean_dec(x_11); if (lean_obj_tag(x_187) == 0) @@ -19107,7 +19585,7 @@ x_194 = lean_box(0); x_195 = lean_box(0); lean_inc(x_7); lean_inc(x_6); -x_196 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___lambda__4(x_11, x_176, x_115, x_111, x_112, x_113, x_195, x_194, x_6, x_7, x_8); +x_196 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___lambda__4(x_11, x_176, x_115, x_111, x_112, x_113, x_195, x_194, x_6, x_7, x_8); lean_dec(x_176); lean_dec(x_11); if (lean_obj_tag(x_196) == 0) @@ -19174,7 +19652,7 @@ if (lean_is_exclusive(x_203)) { } x_208 = lean_box(x_1); lean_inc(x_11); -x_209 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___lambda__1___boxed), 9, 2); +x_209 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___lambda__1___boxed), 9, 2); lean_closure_set(x_209, 0, x_11); lean_closure_set(x_209, 1, x_208); x_210 = l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_typelessBinder_x3f___closed__3; @@ -19190,7 +19668,7 @@ if (x_213 == 0) { lean_object* x_214; uint8_t x_215; lean_dec(x_209); -x_214 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___closed__2; +x_214 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___closed__2; lean_inc(x_11); x_215 = l_Lean_Syntax_isOfKind(x_11, x_214); if (x_215 == 0) @@ -19250,10 +19728,10 @@ x_229 = l_Lean_Syntax_getArg(x_221, x_228); lean_dec(x_221); x_230 = lean_array_size(x_204); x_231 = 0; -x_232 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___closed__3; +x_232 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___closed__3; x_233 = lean_box(0); lean_inc(x_6); -x_234 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5(x_232, x_229, x_204, x_230, x_231, x_233, x_6, x_7, x_8); +x_234 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6(x_232, x_229, x_204, x_230, x_231, x_233, x_6, x_7, x_8); lean_dec(x_229); if (lean_obj_tag(x_234) == 0) { @@ -19360,7 +19838,7 @@ lean_ctor_set(x_255, 0, x_254); x_256 = lean_box(0); lean_inc(x_7); lean_inc(x_6); -x_257 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___lambda__2(x_245, x_209, x_204, x_205, x_206, x_256, x_255, x_6, x_7, x_8); +x_257 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___lambda__2(x_245, x_209, x_204, x_205, x_206, x_256, x_255, x_6, x_7, x_8); lean_dec(x_245); if (lean_obj_tag(x_257) == 0) { @@ -19412,7 +19890,7 @@ x_264 = lean_box(0); x_265 = lean_box(0); lean_inc(x_7); lean_inc(x_6); -x_266 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___lambda__2(x_245, x_209, x_204, x_205, x_206, x_265, x_264, x_6, x_7, x_8); +x_266 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___lambda__2(x_245, x_209, x_204, x_205, x_206, x_265, x_264, x_6, x_7, x_8); lean_dec(x_245); if (lean_obj_tag(x_266) == 0) { @@ -19502,7 +19980,7 @@ lean_ctor_set(x_284, 0, x_283); x_285 = lean_box(0); lean_inc(x_7); lean_inc(x_6); -x_286 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___lambda__4(x_11, x_274, x_209, x_204, x_205, x_206, x_285, x_284, x_6, x_7, x_8); +x_286 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___lambda__4(x_11, x_274, x_209, x_204, x_205, x_206, x_285, x_284, x_6, x_7, x_8); lean_dec(x_274); lean_dec(x_11); if (lean_obj_tag(x_286) == 0) @@ -19554,7 +20032,7 @@ x_293 = lean_box(0); x_294 = lean_box(0); lean_inc(x_7); lean_inc(x_6); -x_295 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___lambda__4(x_11, x_274, x_209, x_204, x_205, x_206, x_294, x_293, x_6, x_7, x_8); +x_295 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___lambda__4(x_11, x_274, x_209, x_204, x_205, x_206, x_294, x_293, x_6, x_7, x_8); lean_dec(x_274); lean_dec(x_11); if (lean_obj_tag(x_295) == 0) @@ -19630,7 +20108,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8(uint8_t 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_mapMUnsafe_map___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__9(uint8_t 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; @@ -19677,12 +20155,12 @@ lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean x_31 = lean_ctor_get(x_29, 1); x_32 = lean_ctor_get(x_29, 0); lean_dec(x_32); -x_33 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__1; +x_33 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__1; lean_inc(x_24); lean_ctor_set_tag(x_29, 2); lean_ctor_set(x_29, 1, x_33); lean_ctor_set(x_29, 0, x_24); -x_34 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__3; +x_34 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__3; lean_inc(x_24); x_35 = l_Lean_Syntax_node1(x_24, x_34, x_10); x_36 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___closed__12; @@ -19691,7 +20169,7 @@ x_37 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_37, 0, x_24); lean_ctor_set(x_37, 1, x_34); lean_ctor_set(x_37, 2, x_36); -x_38 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__4; +x_38 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__4; lean_inc(x_24); lean_ctor_set_tag(x_25, 2); lean_ctor_set(x_25, 1, x_38); @@ -19708,12 +20186,12 @@ lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean x_41 = lean_ctor_get(x_29, 1); lean_inc(x_41); lean_dec(x_29); -x_42 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__1; +x_42 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__1; lean_inc(x_24); x_43 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_43, 0, x_24); lean_ctor_set(x_43, 1, x_42); -x_44 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__3; +x_44 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__3; lean_inc(x_24); x_45 = l_Lean_Syntax_node1(x_24, x_44, x_10); x_46 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___closed__12; @@ -19722,7 +20200,7 @@ x_47 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_47, 0, x_24); lean_ctor_set(x_47, 1, x_44); lean_ctor_set(x_47, 2, x_46); -x_48 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__4; +x_48 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__4; lean_inc(x_24); lean_ctor_set_tag(x_25, 2); lean_ctor_set(x_25, 1, x_48); @@ -19751,7 +20229,7 @@ if (lean_is_exclusive(x_52)) { lean_dec_ref(x_52); x_54 = lean_box(0); } -x_55 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__1; +x_55 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__1; lean_inc(x_24); if (lean_is_scalar(x_54)) { x_56 = lean_alloc_ctor(2, 2, 0); @@ -19761,7 +20239,7 @@ if (lean_is_scalar(x_54)) { } lean_ctor_set(x_56, 0, x_24); lean_ctor_set(x_56, 1, x_55); -x_57 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__3; +x_57 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__3; lean_inc(x_24); x_58 = l_Lean_Syntax_node1(x_24, x_57, x_10); x_59 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___closed__12; @@ -19770,7 +20248,7 @@ x_60 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_60, 0, x_24); lean_ctor_set(x_60, 1, x_57); lean_ctor_set(x_60, 2, x_59); -x_61 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__4; +x_61 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__4; lean_inc(x_24); x_62 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_62, 0, x_24); @@ -19810,12 +20288,12 @@ lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean x_76 = lean_ctor_get(x_74, 1); x_77 = lean_ctor_get(x_74, 0); lean_dec(x_77); -x_78 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__6; +x_78 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__6; lean_inc(x_69); lean_ctor_set_tag(x_74, 2); lean_ctor_set(x_74, 1, x_78); lean_ctor_set(x_74, 0, x_69); -x_79 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__3; +x_79 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__3; lean_inc(x_69); x_80 = l_Lean_Syntax_node1(x_69, x_79, x_10); x_81 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___closed__12; @@ -19842,12 +20320,12 @@ lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean x_86 = lean_ctor_get(x_74, 1); lean_inc(x_86); lean_dec(x_74); -x_87 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__6; +x_87 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__6; 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_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__3; +x_89 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__3; lean_inc(x_69); x_90 = l_Lean_Syntax_node1(x_69, x_89, x_10); x_91 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___closed__12; @@ -19886,7 +20364,7 @@ if (lean_is_exclusive(x_97)) { lean_dec_ref(x_97); x_99 = lean_box(0); } -x_100 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__6; +x_100 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__6; lean_inc(x_69); if (lean_is_scalar(x_99)) { x_101 = lean_alloc_ctor(2, 2, 0); @@ -19896,7 +20374,7 @@ if (lean_is_scalar(x_99)) { } lean_ctor_set(x_101, 0, x_69); lean_ctor_set(x_101, 1, x_100); -x_102 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__3; +x_102 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__3; lean_inc(x_69); x_103 = l_Lean_Syntax_node1(x_69, x_102, x_10); x_104 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___closed__12; @@ -19945,7 +20423,7 @@ size_t x_13; lean_object* x_14; lean_dec(x_6); lean_dec(x_5); x_13 = lean_array_size(x_1); -x_14 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8(x_3, x_13, x_4, x_1, x_8, x_9, x_10); +x_14 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__9(x_3, x_13, x_4, x_1, x_8, x_9, x_10); return x_14; } else @@ -20080,7 +20558,7 @@ x_23 = 0; x_24 = lean_unbox(x_12); lean_inc(x_3); lean_inc(x_2); -x_25 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7(x_24, x_20, x_22, x_23, x_13, x_2, x_3, x_16); +x_25 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8(x_24, x_20, x_22, x_23, x_13, x_2, x_3, x_16); lean_dec(x_20); if (lean_obj_tag(x_25) == 0) { @@ -20193,7 +20671,7 @@ x_57 = 0; x_58 = lean_unbox(x_12); lean_inc(x_3); lean_inc(x_2); -x_59 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7(x_58, x_53, x_56, x_57, x_55, x_2, x_3, x_49); +x_59 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8(x_58, x_53, x_56, x_57, x_55, x_2, x_3, x_49); lean_dec(x_53); if (lean_obj_tag(x_59) == 0) { @@ -20288,6 +20766,15 @@ return x_81; } } } +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___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___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__2(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; +} +} LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { @@ -20298,7 +20785,7 @@ lean_dec(x_1); return x_6; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___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: { size_t x_9; size_t x_10; lean_object* x_11; @@ -20306,14 +20793,14 @@ x_9 = lean_unbox_usize(x_3); lean_dec(x_3); x_10 = lean_unbox_usize(x_4); lean_dec(x_4); -x_11 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__2(x_1, x_2, x_9, x_10, x_5, x_6, x_7, x_8); +x_11 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__3(x_1, x_2, x_9, x_10, x_5, x_6, x_7, x_8); lean_dec(x_7); lean_dec(x_2); lean_dec(x_1); return x_11; } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___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_anyMUnsafe_any___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___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; @@ -20321,25 +20808,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_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__3(x_1, x_2, x_5, x_6); +x_7 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4(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___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___lambda__1(x_1, x_2); +x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___lambda__1(x_1, x_2); lean_dec(x_2); lean_dec(x_1); x_4 = lean_box(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___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_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___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: { uint8_t x_11; uint8_t x_12; size_t x_13; size_t x_14; lean_object* x_15; @@ -20351,14 +20838,14 @@ x_13 = lean_unbox_usize(x_5); lean_dec(x_5); x_14 = lean_unbox_usize(x_6); lean_dec(x_6); -x_15 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4(x_11, x_2, x_12, x_4, x_13, x_14, x_7, x_8, x_9, x_10); +x_15 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5(x_11, x_2, x_12, x_4, x_13, x_14, x_7, x_8, x_9, x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_4); return x_15; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { size_t x_10; size_t x_11; lean_object* x_12; @@ -20366,7 +20853,7 @@ x_10 = lean_unbox_usize(x_4); lean_dec(x_4); x_11 = lean_unbox_usize(x_5); lean_dec(x_5); -x_12 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5(x_1, x_2, x_3, x_10, x_11, x_6, x_7, x_8, x_9); +x_12 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6(x_1, x_2, x_3, x_10, x_11, x_6, x_7, x_8, x_9); lean_dec(x_8); lean_dec(x_3); lean_dec(x_2); @@ -20374,7 +20861,7 @@ lean_dec(x_1); return x_12; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { size_t x_9; size_t x_10; lean_object* x_11; @@ -20382,14 +20869,14 @@ x_9 = lean_unbox_usize(x_3); lean_dec(x_3); x_10 = lean_unbox_usize(x_4); lean_dec(x_4); -x_11 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6(x_1, x_2, x_9, x_10, x_5, x_6, x_7, x_8); +x_11 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7(x_1, x_2, x_9, x_10, x_5, x_6, x_7, x_8); lean_dec(x_7); lean_dec(x_2); lean_dec(x_1); return x_11; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___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_object* x_9) { _start: { uint8_t x_10; uint8_t x_11; lean_object* x_12; @@ -20397,42 +20884,42 @@ x_10 = lean_unbox(x_2); lean_dec(x_2); x_11 = lean_unbox(x_4); lean_dec(x_4); -x_12 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___lambda__1(x_1, x_10, x_3, x_11, x_5, x_6, x_7, x_8, x_9); +x_12 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___lambda__1(x_1, x_10, x_3, x_11, x_5, x_6, x_7, x_8, x_9); lean_dec(x_8); return x_12; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; -x_11 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___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_6); lean_dec(x_1); return x_11; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; -x_11 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___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); return x_11; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_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_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { lean_object* x_12; -x_12 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_12 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_7); lean_dec(x_2); lean_dec(x_1); return x_12; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___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: { uint8_t x_9; size_t x_10; size_t x_11; lean_object* x_12; @@ -20442,12 +20929,12 @@ x_10 = lean_unbox_usize(x_3); lean_dec(x_3); x_11 = lean_unbox_usize(x_4); lean_dec(x_4); -x_12 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7(x_9, x_2, x_10, x_11, x_5, x_6, x_7, x_8); +x_12 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8(x_9, x_2, x_10, x_11, x_5, x_6, x_7, x_8); lean_dec(x_2); return x_12; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___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_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___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) { _start: { uint8_t x_8; size_t x_9; size_t x_10; lean_object* x_11; @@ -20457,7 +20944,7 @@ x_9 = lean_unbox_usize(x_2); lean_dec(x_2); x_10 = lean_unbox_usize(x_3); lean_dec(x_3); -x_11 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8(x_8, x_9, x_10, x_4, x_5, x_6, x_7); +x_11 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__9(x_8, x_9, x_10, x_4, x_5, x_6, x_7); lean_dec(x_6); lean_dec(x_5); return x_11; @@ -21674,7 +22161,7 @@ lean_inc(x_39); x_40 = lean_ctor_get(x_38, 1); lean_inc(x_40); lean_dec(x_38); -x_41 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__1; +x_41 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__1; x_42 = l_Lean_Elab_Term_levelMVarToParam(x_39, x_41, x_5, x_6, x_7, x_8, x_9, x_10, x_40); x_43 = !lean_is_exclusive(x_42); if (x_43 == 0) @@ -22588,7 +23075,7 @@ lean_inc(x_40); x_41 = lean_ctor_get(x_39, 1); lean_inc(x_41); lean_dec(x_39); -x_42 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__1; +x_42 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__1; x_43 = l_Lean_Elab_Term_levelMVarToParam(x_40, x_42, x_6, x_7, x_8, x_9, x_10, x_11, x_41); x_44 = !lean_is_exclusive(x_10); if (x_44 == 0) @@ -25479,7 +25966,7 @@ lean_inc(x_17); x_19 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_19, 0, x_17); lean_ctor_set(x_19, 1, x_18); -x_20 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__3; +x_20 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__3; x_21 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___closed__12; lean_inc(x_17); x_22 = lean_alloc_ctor(1, 3, 0); @@ -25950,119 +26437,345 @@ return x_28; } } } -LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAddDeclDoc___spec__6(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_addDocString___at_Lean_Elab_Command_elabAddDeclDoc___spec__5___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; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_8 = lean_ctor_get(x_6, 0); -x_9 = lean_ctor_get(x_6, 1); -x_10 = lean_ctor_get(x_8, 0); -lean_inc(x_10); -lean_dec(x_8); -x_11 = l_Lean_instInhabitedDeclarationRanges; -x_12 = l_Lean_findDeclarationRangesCore_x3f___at_Lean_Elab_Command_elabAddDeclDoc___spec__1___closed__1; -lean_inc(x_1); -x_13 = l_Lean_MapDeclarationExtension_contains___rarg(x_11, x_12, x_10, x_1); -lean_dec(x_10); -if (x_13 == 0) +lean_object* x_1; +x_1 = l_Lean_docStringExt; +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_addDocString___at_Lean_Elab_Command_elabAddDeclDoc___spec__5___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: { -lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; -lean_free_object(x_6); -x_14 = lean_st_ref_take(x_4, 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 = !lean_is_exclusive(x_15); -if (x_17 == 0) +lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; +x_7 = lean_st_ref_take(x_5, x_6); +x_8 = lean_ctor_get(x_7, 0); +lean_inc(x_8); +x_9 = lean_ctor_get(x_7, 1); +lean_inc(x_9); +lean_dec(x_7); +x_10 = !lean_is_exclusive(x_8); +if (x_10 == 0) { -lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; -x_18 = lean_ctor_get(x_15, 0); -x_19 = l_Lean_MapDeclarationExtension_insert___rarg(x_12, x_18, x_1, x_2); -lean_ctor_set(x_15, 0, x_19); -x_20 = lean_st_ref_set(x_4, x_15, x_16); -x_21 = !lean_is_exclusive(x_20); -if (x_21 == 0) +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_11 = lean_ctor_get(x_8, 0); +x_12 = l_String_removeLeadingSpaces(x_1); +x_13 = l_Lean_addDocString___at_Lean_Elab_Command_elabAddDeclDoc___spec__5___lambda__1___closed__1; +x_14 = l_Lean_MapDeclarationExtension_insert___rarg(x_13, x_11, x_2, x_12); +lean_ctor_set(x_8, 0, x_14); +x_15 = lean_st_ref_set(x_5, x_8, x_9); +x_16 = !lean_is_exclusive(x_15); +if (x_16 == 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; +lean_object* x_17; lean_object* x_18; +x_17 = lean_ctor_get(x_15, 0); +lean_dec(x_17); +x_18 = lean_box(0); +lean_ctor_set(x_15, 0, x_18); +return x_15; } else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_20, 1); -lean_inc(x_24); -lean_dec(x_20); -x_25 = lean_box(0); -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_26, 1, x_24); -return x_26; +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_15, 1); +lean_inc(x_19); +lean_dec(x_15); +x_20 = lean_box(0); +x_21 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_21, 0, x_20); +lean_ctor_set(x_21, 1, x_19); +return x_21; } } else { -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; -x_27 = lean_ctor_get(x_15, 0); -x_28 = lean_ctor_get(x_15, 1); -x_29 = lean_ctor_get(x_15, 2); -x_30 = lean_ctor_get(x_15, 3); -x_31 = lean_ctor_get(x_15, 4); -x_32 = lean_ctor_get(x_15, 5); -x_33 = lean_ctor_get(x_15, 6); -x_34 = lean_ctor_get(x_15, 7); -lean_inc(x_34); -lean_inc(x_33); -lean_inc(x_32); -lean_inc(x_31); -lean_inc(x_30); +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_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_22 = lean_ctor_get(x_8, 0); +x_23 = lean_ctor_get(x_8, 1); +x_24 = lean_ctor_get(x_8, 2); +x_25 = lean_ctor_get(x_8, 3); +x_26 = lean_ctor_get(x_8, 4); +x_27 = lean_ctor_get(x_8, 5); +x_28 = lean_ctor_get(x_8, 6); +x_29 = lean_ctor_get(x_8, 7); lean_inc(x_29); lean_inc(x_28); lean_inc(x_27); -lean_dec(x_15); -x_35 = l_Lean_MapDeclarationExtension_insert___rarg(x_12, x_27, x_1, x_2); -x_36 = lean_alloc_ctor(0, 8, 0); -lean_ctor_set(x_36, 0, x_35); -lean_ctor_set(x_36, 1, x_28); -lean_ctor_set(x_36, 2, x_29); -lean_ctor_set(x_36, 3, x_30); -lean_ctor_set(x_36, 4, x_31); -lean_ctor_set(x_36, 5, x_32); -lean_ctor_set(x_36, 6, x_33); -lean_ctor_set(x_36, 7, x_34); -x_37 = lean_st_ref_set(x_4, x_36, x_16); -x_38 = lean_ctor_get(x_37, 1); -lean_inc(x_38); -if (lean_is_exclusive(x_37)) { - lean_ctor_release(x_37, 0); - lean_ctor_release(x_37, 1); - x_39 = x_37; +lean_inc(x_26); +lean_inc(x_25); +lean_inc(x_24); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_8); +x_30 = l_String_removeLeadingSpaces(x_1); +x_31 = l_Lean_addDocString___at_Lean_Elab_Command_elabAddDeclDoc___spec__5___lambda__1___closed__1; +x_32 = l_Lean_MapDeclarationExtension_insert___rarg(x_31, x_22, x_2, x_30); +x_33 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_23); +lean_ctor_set(x_33, 2, x_24); +lean_ctor_set(x_33, 3, x_25); +lean_ctor_set(x_33, 4, x_26); +lean_ctor_set(x_33, 5, x_27); +lean_ctor_set(x_33, 6, x_28); +lean_ctor_set(x_33, 7, x_29); +x_34 = lean_st_ref_set(x_5, x_33, x_9); +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_37); - x_39 = lean_box(0); + lean_dec_ref(x_34); + x_36 = lean_box(0); } -x_40 = lean_box(0); -if (lean_is_scalar(x_39)) { - x_41 = 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_41 = x_39; + x_38 = x_36; } -lean_ctor_set(x_41, 0, x_40); -lean_ctor_set(x_41, 1, x_38); -return x_41; +lean_ctor_set(x_38, 0, x_37); +lean_ctor_set(x_38, 1, x_35); +return x_38; } } -else +} +static lean_object* _init_l_Lean_addDocString___at_Lean_Elab_Command_elabAddDeclDoc___spec__5___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("invalid doc string, declaration '", 33, 33); +return x_1; +} +} +static lean_object* _init_l_Lean_addDocString___at_Lean_Elab_Command_elabAddDeclDoc___spec__5___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("' is in an imported module", 26, 26); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_addDocString___at_Lean_Elab_Command_elabAddDeclDoc___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_6 = lean_st_ref_get(x_4, x_5); +x_7 = lean_ctor_get(x_6, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_6, 1); +lean_inc(x_8); +lean_dec(x_6); +x_9 = lean_ctor_get(x_7, 0); +lean_inc(x_9); +lean_dec(x_7); +x_10 = l_Lean_Environment_getModuleIdxFor_x3f(x_9, x_1); +lean_dec(x_9); +if (lean_obj_tag(x_10) == 0) +{ +lean_object* x_11; lean_object* x_12; +x_11 = lean_box(0); +x_12 = l_Lean_addDocString___at_Lean_Elab_Command_elabAddDeclDoc___spec__5___lambda__1(x_2, x_1, x_11, x_3, x_4, x_8); +lean_dec(x_3); +return x_12; +} +else +{ +uint8_t x_13; +lean_dec(x_2); +x_13 = !lean_is_exclusive(x_10); +if (x_13 == 0) +{ +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; uint8_t x_24; +x_14 = lean_ctor_get(x_10, 0); +lean_dec(x_14); +x_15 = 1; +x_16 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__1; +x_17 = l_Lean_Name_toString(x_1, x_15, x_16); +x_18 = l_Lean_addDocString___at_Lean_Elab_Command_elabAddDeclDoc___spec__5___closed__1; +x_19 = lean_string_append(x_18, x_17); +lean_dec(x_17); +x_20 = l_Lean_addDocString___at_Lean_Elab_Command_elabAddDeclDoc___spec__5___closed__2; +x_21 = lean_string_append(x_19, x_20); +lean_ctor_set_tag(x_10, 3); +lean_ctor_set(x_10, 0, x_21); +x_22 = l_Lean_MessageData_ofFormat(x_10); +x_23 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__7(x_22, x_3, x_4, x_8); +x_24 = !lean_is_exclusive(x_23); +if (x_24 == 0) +{ +return x_23; +} +else +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_23, 0); +x_26 = lean_ctor_get(x_23, 1); +lean_inc(x_26); +lean_inc(x_25); +lean_dec(x_23); +x_27 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +return x_27; +} +} +else +{ +uint8_t x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; +lean_dec(x_10); +x_28 = 1; +x_29 = l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__1; +x_30 = l_Lean_Name_toString(x_1, x_28, x_29); +x_31 = l_Lean_addDocString___at_Lean_Elab_Command_elabAddDeclDoc___spec__5___closed__1; +x_32 = lean_string_append(x_31, x_30); +lean_dec(x_30); +x_33 = l_Lean_addDocString___at_Lean_Elab_Command_elabAddDeclDoc___spec__5___closed__2; +x_34 = lean_string_append(x_32, x_33); +x_35 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_35, 0, x_34); +x_36 = l_Lean_MessageData_ofFormat(x_35); +x_37 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__7(x_36, x_3, x_4, x_8); +x_38 = lean_ctor_get(x_37, 0); +lean_inc(x_38); +x_39 = lean_ctor_get(x_37, 1); +lean_inc(x_39); +if (lean_is_exclusive(x_37)) { + lean_ctor_release(x_37, 0); + lean_ctor_release(x_37, 1); + x_40 = x_37; +} else { + lean_dec_ref(x_37); + x_40 = lean_box(0); +} +if (lean_is_scalar(x_40)) { + x_41 = lean_alloc_ctor(1, 2, 0); +} else { + x_41 = x_40; +} +lean_ctor_set(x_41, 0, x_38); +lean_ctor_set(x_41, 1, x_39); +return x_41; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAddDeclDoc___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; uint8_t x_7; +x_6 = lean_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; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_8 = lean_ctor_get(x_6, 0); +x_9 = lean_ctor_get(x_6, 1); +x_10 = lean_ctor_get(x_8, 0); +lean_inc(x_10); +lean_dec(x_8); +x_11 = l_Lean_instInhabitedDeclarationRanges; +x_12 = l_Lean_findDeclarationRangesCore_x3f___at_Lean_Elab_Command_elabAddDeclDoc___spec__1___closed__1; +lean_inc(x_1); +x_13 = l_Lean_MapDeclarationExtension_contains___rarg(x_11, x_12, x_10, x_1); +lean_dec(x_10); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +lean_free_object(x_6); +x_14 = lean_st_ref_take(x_4, 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 = !lean_is_exclusive(x_15); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_18 = lean_ctor_get(x_15, 0); +x_19 = l_Lean_MapDeclarationExtension_insert___rarg(x_12, x_18, x_1, x_2); +lean_ctor_set(x_15, 0, x_19); +x_20 = lean_st_ref_set(x_4, x_15, x_16); +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; lean_object* x_40; lean_object* x_41; +x_27 = lean_ctor_get(x_15, 0); +x_28 = lean_ctor_get(x_15, 1); +x_29 = lean_ctor_get(x_15, 2); +x_30 = lean_ctor_get(x_15, 3); +x_31 = lean_ctor_get(x_15, 4); +x_32 = lean_ctor_get(x_15, 5); +x_33 = lean_ctor_get(x_15, 6); +x_34 = lean_ctor_get(x_15, 7); +lean_inc(x_34); +lean_inc(x_33); +lean_inc(x_32); +lean_inc(x_31); +lean_inc(x_30); +lean_inc(x_29); +lean_inc(x_28); +lean_inc(x_27); +lean_dec(x_15); +x_35 = l_Lean_MapDeclarationExtension_insert___rarg(x_12, x_27, x_1, x_2); +x_36 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_36, 0, x_35); +lean_ctor_set(x_36, 1, x_28); +lean_ctor_set(x_36, 2, x_29); +lean_ctor_set(x_36, 3, x_30); +lean_ctor_set(x_36, 4, x_31); +lean_ctor_set(x_36, 5, x_32); +lean_ctor_set(x_36, 6, x_33); +lean_ctor_set(x_36, 7, x_34); +x_37 = lean_st_ref_set(x_4, x_36, x_16); +x_38 = lean_ctor_get(x_37, 1); +lean_inc(x_38); +if (lean_is_exclusive(x_37)) { + lean_ctor_release(x_37, 0); + lean_ctor_release(x_37, 1); + x_39 = x_37; +} else { + lean_dec_ref(x_37); + x_39 = lean_box(0); +} +x_40 = lean_box(0); +if (lean_is_scalar(x_39)) { + x_41 = lean_alloc_ctor(0, 2, 0); +} else { + x_41 = x_39; +} +lean_ctor_set(x_41, 0, x_40); +lean_ctor_set(x_41, 1, x_38); +return x_41; +} +} +else { lean_object* x_42; lean_dec(x_2); @@ -26176,85 +26889,163 @@ return x_69; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___at_Lean_Elab_Command_elabAddDeclDoc___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___at_Lean_Elab_Command_elabAddDeclDoc___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: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; +lean_object* x_7; lean_object* x_8; lean_inc(x_4); -x_7 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Command_elabModuleDoc___spec__2(x_2, x_4, x_5, x_6); +x_7 = l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Command_elabModuleDoc___spec__2(x_2, x_4, x_5, x_6); x_8 = lean_ctor_get(x_7, 0); lean_inc(x_8); -x_9 = lean_ctor_get(x_7, 1); -lean_inc(x_9); -lean_dec(x_7); -lean_inc(x_4); -x_10 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Command_elabModuleDoc___spec__2(x_3, x_4, x_5, x_9); -x_11 = !lean_is_exclusive(x_10); -if (x_11 == 0) +if (lean_obj_tag(x_8) == 0) { -lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_12 = lean_ctor_get(x_10, 0); -x_13 = lean_ctor_get(x_10, 1); -lean_ctor_set(x_10, 1, x_12); -lean_ctor_set(x_10, 0, x_8); -x_14 = l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAddDeclDoc___spec__6(x_1, x_10, x_4, x_5, x_13); +uint8_t x_9; lean_dec(x_4); -return x_14; -} -else +lean_dec(x_1); +x_9 = !lean_is_exclusive(x_7); +if (x_9 == 0) { -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_15 = lean_ctor_get(x_10, 0); -x_16 = lean_ctor_get(x_10, 1); -lean_inc(x_16); -lean_inc(x_15); +lean_object* x_10; lean_object* x_11; +x_10 = lean_ctor_get(x_7, 0); lean_dec(x_10); -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_8); -lean_ctor_set(x_17, 1, x_15); -x_18 = l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAddDeclDoc___spec__6(x_1, x_17, x_4, x_5, x_16); -lean_dec(x_4); -return x_18; -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAddDeclDoc___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -lean_object* x_7; -lean_inc(x_4); -x_7 = l_Lean_getDocStringText___at_Lean_Elab_Command_elabAddDeclDoc___spec__2(x_1, x_4, x_5, x_6); -if (lean_obj_tag(x_7) == 0) -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; -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_addDocString___at_Lean_Elab_Command_expandDeclId___spec__14(x_2, x_8, x_4, x_5, x_9); -return x_10; -} -else -{ -uint8_t x_11; -lean_dec(x_4); -lean_dec(x_2); -x_11 = !lean_is_exclusive(x_7); -if (x_11 == 0) -{ +x_11 = lean_box(0); +lean_ctor_set(x_7, 0, x_11); return x_7; } else { lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_12 = lean_ctor_get(x_7, 0); -x_13 = lean_ctor_get(x_7, 1); -lean_inc(x_13); +x_12 = lean_ctor_get(x_7, 1); lean_inc(x_12); lean_dec(x_7); -x_14 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_14, 0, 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); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_15 = lean_ctor_get(x_7, 1); +lean_inc(x_15); +lean_dec(x_7); +x_16 = lean_ctor_get(x_8, 0); +lean_inc(x_16); +lean_dec(x_8); +lean_inc(x_4); +x_17 = l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Command_elabModuleDoc___spec__2(x_3, x_4, x_5, x_15); +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +if (lean_obj_tag(x_18) == 0) +{ +uint8_t x_19; +x_19 = !lean_is_exclusive(x_17); +if (x_19 == 0) +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_17, 1); +x_21 = lean_ctor_get(x_17, 0); +lean_dec(x_21); +lean_inc(x_16); +lean_ctor_set(x_17, 1, x_16); +lean_ctor_set(x_17, 0, x_16); +x_22 = l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAddDeclDoc___spec__7(x_1, x_17, x_4, x_5, x_20); +lean_dec(x_4); +return x_22; +} +else +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_17, 1); +lean_inc(x_23); +lean_dec(x_17); +lean_inc(x_16); +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_16); +lean_ctor_set(x_24, 1, x_16); +x_25 = l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAddDeclDoc___spec__7(x_1, x_24, x_4, x_5, x_23); +lean_dec(x_4); +return x_25; +} +} +else +{ +uint8_t x_26; +x_26 = !lean_is_exclusive(x_17); +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_17, 1); +x_28 = lean_ctor_get(x_17, 0); +lean_dec(x_28); +x_29 = lean_ctor_get(x_18, 0); +lean_inc(x_29); +lean_dec(x_18); +lean_ctor_set(x_17, 1, x_29); +lean_ctor_set(x_17, 0, x_16); +x_30 = l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAddDeclDoc___spec__7(x_1, x_17, x_4, x_5, x_27); +lean_dec(x_4); +return x_30; +} +else +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_31 = lean_ctor_get(x_17, 1); +lean_inc(x_31); +lean_dec(x_17); +x_32 = lean_ctor_get(x_18, 0); +lean_inc(x_32); +lean_dec(x_18); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_16); +lean_ctor_set(x_33, 1, x_32); +x_34 = l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAddDeclDoc___spec__7(x_1, x_33, x_4, x_5, x_31); +lean_dec(x_4); +return x_34; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAddDeclDoc___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; +lean_inc(x_4); +x_7 = l_Lean_getDocStringText___at_Lean_Elab_Command_elabAddDeclDoc___spec__2(x_1, x_4, x_5, x_6); +if (lean_obj_tag(x_7) == 0) +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; +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_addDocString___at_Lean_Elab_Command_elabAddDeclDoc___spec__5(x_2, x_8, x_4, x_5, x_9); +return x_10; +} +else +{ +uint8_t x_11; +lean_dec(x_4); +lean_dec(x_2); +x_11 = !lean_is_exclusive(x_7); +if (x_11 == 0) +{ +return x_7; +} +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_7, 0); +x_13 = lean_ctor_get(x_7, 1); +lean_inc(x_13); +lean_inc(x_12); +lean_dec(x_7); +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; } @@ -26277,7 +27068,7 @@ lean_inc(x_11); lean_dec(x_9); lean_inc(x_6); lean_inc(x_1); -x_12 = l_Lean_Elab_addAuxDeclarationRanges___at_Lean_Elab_Command_elabAddDeclDoc___spec__5(x_1, x_3, x_4, x_6, x_7, x_11); +x_12 = l_Lean_Elab_addDeclarationRangesFromSyntax___at_Lean_Elab_Command_elabAddDeclDoc___spec__6(x_1, x_3, x_4, x_6, x_7, x_11); x_13 = lean_ctor_get(x_12, 0); lean_inc(x_13); x_14 = lean_ctor_get(x_12, 1); @@ -26438,7 +27229,7 @@ lean_dec(x_14); lean_dec(x_9); lean_dec(x_1); x_27 = l_Lean_Elab_Command_elabAddDeclDoc___closed__6; -x_28 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_27, x_2, x_3, x_22); +x_28 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__7(x_27, x_2, x_3, x_22); x_29 = !lean_is_exclusive(x_28); if (x_29 == 0) { @@ -26528,21 +27319,41 @@ lean_dec(x_1); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAddDeclDoc___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_addDocString___at_Lean_Elab_Command_elabAddDeclDoc___spec__5___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; +x_7 = l_Lean_addDocString___at_Lean_Elab_Command_elabAddDeclDoc___spec__5___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_addDocString___at_Lean_Elab_Command_elabAddDeclDoc___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_Lean_addDocString___at_Lean_Elab_Command_elabAddDeclDoc___spec__5(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_4); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAddDeclDoc___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; -x_6 = l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAddDeclDoc___spec__6(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAddDeclDoc___spec__7(x_1, x_2, x_3, x_4, x_5); lean_dec(x_4); lean_dec(x_3); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___at_Lean_Elab_Command_elabAddDeclDoc___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___at_Lean_Elab_Command_elabAddDeclDoc___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) { _start: { lean_object* x_7; -x_7 = l_Lean_Elab_addAuxDeclarationRanges___at_Lean_Elab_Command_elabAddDeclDoc___spec__5(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Lean_Elab_addDeclarationRangesFromSyntax___at_Lean_Elab_Command_elabAddDeclDoc___spec__6(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_5); lean_dec(x_3); lean_dec(x_2); @@ -26804,7 +27615,7 @@ x_19 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInclude___spec__1___c x_20 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_20, 0, x_18); lean_ctor_set(x_20, 1, x_19); -x_21 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__18(x_20, x_7, x_8, x_9); +x_21 = l_Lean_throwError___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__2(x_20, x_7, x_8, x_9); x_22 = !lean_is_exclusive(x_21); if (x_22 == 0) { @@ -26882,7 +27693,7 @@ if (x_5 == 0) lean_object* x_6; lean_object* x_7; uint8_t x_8; x_6 = lean_ctor_get(x_2, 0); x_7 = lean_ctor_get(x_2, 1); -x_8 = l_Array_contains___at_Lean_findField_x3f___spec__1(x_1, x_6); +x_8 = l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(x_1, x_6); if (x_8 == 0) { lean_ctor_set(x_2, 1, x_3); @@ -26910,7 +27721,7 @@ x_12 = lean_ctor_get(x_2, 1); lean_inc(x_12); lean_inc(x_11); lean_dec(x_2); -x_13 = l_Array_contains___at_Lean_findField_x3f___spec__1(x_1, x_11); +x_13 = l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(x_1, x_11); if (x_13 == 0) { lean_object* x_14; @@ -28503,7 +29314,7 @@ if (x_25 == 0) lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; lean_dec(x_4); x_28 = l_Lean_MessageData_ofSyntax(x_14); -x_29 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__11___closed__3; +x_29 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__12___closed__3; x_30 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_30, 0, x_29); lean_ctor_set(x_30, 1, x_28); @@ -28560,7 +29371,7 @@ if (x_42 == 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_dec(x_45); x_46 = l_Lean_MessageData_ofSyntax(x_14); -x_47 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__11___closed__3; +x_47 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__12___closed__3; x_48 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_48, 0, x_47); lean_ctor_set(x_48, 1, x_46); @@ -28825,7 +29636,7 @@ if (x_5 == 0) lean_object* x_6; lean_object* x_7; uint8_t x_8; x_6 = lean_ctor_get(x_2, 0); x_7 = lean_ctor_get(x_2, 1); -x_8 = l_Array_contains___at_Lean_findField_x3f___spec__1(x_1, x_6); +x_8 = l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(x_1, x_6); if (x_8 == 0) { lean_ctor_set(x_2, 1, x_3); @@ -28853,7 +29664,7 @@ x_12 = lean_ctor_get(x_2, 1); lean_inc(x_12); lean_inc(x_11); lean_dec(x_2); -x_13 = l_Array_contains___at_Lean_findField_x3f___spec__1(x_1, x_11); +x_13 = l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(x_1, x_11); if (x_13 == 0) { lean_object* x_14; @@ -29235,300 +30046,1003 @@ x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabOmit(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabOmit(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; uint8_t x_6; +x_5 = l_Lean_Elab_Command_elabOmit___closed__2; +lean_inc(x_1); +x_6 = l_Lean_Syntax_isOfKind(x_1, x_5); +if (x_6 == 0) +{ +lean_object* x_7; +lean_dec(x_1); +x_7 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabNamespace___spec__1___rarg(x_4); +return x_7; +} +else +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_8 = lean_unsigned_to_nat(1u); +x_9 = l_Lean_Syntax_getArg(x_1, x_8); +lean_dec(x_1); +x_10 = lean_box(0); +x_11 = l_Lean_Syntax_getArgs(x_9); +lean_dec(x_9); +x_12 = l_Lean_Elab_Command_elabSection___closed__4; +x_13 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___closed__2; +x_14 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabOmit___lambda__1___boxed), 12, 4); +lean_closure_set(x_14, 0, x_11); +lean_closure_set(x_14, 1, x_12); +lean_closure_set(x_14, 2, x_13); +lean_closure_set(x_14, 3, x_10); +x_15 = l_Lean_Elab_Command_runTermElabM___rarg(x_14, x_2, x_3, x_4); +if (lean_obj_tag(x_15) == 0) +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_15, 1); +lean_inc(x_17); +lean_dec(x_15); +x_18 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabOmit___lambda__2), 3, 2); +lean_closure_set(x_18, 0, x_16); +lean_closure_set(x_18, 1, x_10); +x_19 = l_Lean_Elab_Command_modifyScope(x_18, x_2, x_3, x_17); +return x_19; +} +else +{ +uint8_t x_20; +x_20 = !lean_is_exclusive(x_15); +if (x_20 == 0) +{ +return x_15; +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_15, 0); +x_22 = lean_ctor_get(x_15, 1); +lean_inc(x_22); +lean_inc(x_21); +lean_dec(x_15); +x_23 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_23, 0, x_21); +lean_ctor_set(x_23, 1, x_22); +return x_23; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabOmit___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; +x_7 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabOmit___spec__1(x_1, x_2, x_3, x_4, x_5, x_6); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabOmit___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +size_t x_14; size_t x_15; lean_object* x_16; +x_14 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_15 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_16 = l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabOmit___spec__3(x_1, x_2, x_3, x_14, x_15, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_16; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabOmit___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; size_t x_5; lean_object* x_6; +x_4 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabOmit___spec__4(x_4, x_5, x_3); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Elab_Command_elabOmit___spec__5___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +uint8_t x_3; lean_object* x_4; +x_3 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Elab_Command_elabOmit___spec__5(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +x_4 = lean_box(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Elab_Command_elabOmit___spec__10___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Elab_Command_elabOmit___spec__10(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__11___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__11___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +size_t x_14; size_t x_15; lean_object* x_16; +x_14 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_15 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_16 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__11(x_1, x_2, x_3, x_14, x_15, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_1); +return x_16; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__12___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__12___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__12___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +size_t x_15; size_t x_16; size_t x_17; lean_object* x_18; +x_15 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_16 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_17 = lean_unbox_usize(x_6); +lean_dec(x_6); +x_18 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__12(x_15, x_2, x_3, x_4, x_16, x_17, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_9); +lean_dec(x_4); +lean_dec(x_2); +return x_18; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +size_t x_12; size_t x_13; lean_object* x_14; +x_12 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_13 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_14 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__13(x_1, x_12, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_1); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at_Lean_Elab_Command_elabOmit___spec__14___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_RBNode_forIn_visit___at_Lean_Elab_Command_elabOmit___spec__14(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_11; +} +} +LEAN_EXPORT lean_object* l_List_filterTR_loop___at_Lean_Elab_Command_elabOmit___spec__15___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_List_filterTR_loop___at_Lean_Elab_Command_elabOmit___spec__15(x_1, x_2, x_3); +lean_dec(x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabOmit___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; +x_13 = l_Lean_Elab_Command_elabOmit___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabOmit___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Lean_Elab_Command_elabOmit(x_1, x_2, x_3, x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_5; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabOmit__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("elabOmit", 8, 8); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabOmit__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l___regBuiltin_Lean_Elab_Command_elabModuleDoc__1___closed__1; +x_2 = l___regBuiltin_Lean_Elab_Command_elabModuleDoc__1___closed__6; +x_3 = l___regBuiltin_Lean_Elab_Command_elabModuleDoc__1___closed__3; +x_4 = l___regBuiltin_Lean_Elab_Command_elabOmit__1___closed__1; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabOmit__1___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabOmit___boxed), 4, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabOmit__1(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Elab_Command_elabModuleDoc__1___closed__9; +x_3 = l_Lean_Elab_Command_elabOmit___closed__2; +x_4 = l___regBuiltin_Lean_Elab_Command_elabOmit__1___closed__2; +x_5 = l___regBuiltin_Lean_Elab_Command_elabOmit__1___closed__3; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean ", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_versionString; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__2; +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__3; +x_3 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("\nTarget: ", 9, 9); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__5; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__4; +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__6; +x_3 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = l_List_appendTR___rarg(x_1, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__9() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__8; +x_3 = l_List_appendTR___rarg(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_elabModuleDoc___closed__3; +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__9; +x_3 = l_List_foldl___at_String_join___spec__1(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__11() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__10; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__12() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" Emscripten", 11, 11); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__13() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__12; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__14() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__8; +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__13; +x_3 = l_List_appendTR___rarg(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__15() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_elabModuleDoc___closed__3; +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__14; +x_3 = l_List_foldl___at_String_join___spec__1(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__16() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__15; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__17() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" macOS", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__18() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__17; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__19() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__18; +x_3 = l_List_appendTR___rarg(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__20() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__19; +x_3 = l_List_appendTR___rarg(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__21() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_elabModuleDoc___closed__3; +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__20; +x_3 = l_List_foldl___at_String_join___spec__1(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__22() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__21; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__23() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__19; +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__13; +x_3 = l_List_appendTR___rarg(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__24() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_elabModuleDoc___closed__3; +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__23; +x_3 = l_List_foldl___at_String_join___spec__1(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__25() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__24; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__26() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" Windows", 8, 8); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__27() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__26; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__28() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__27; +x_3 = l_List_appendTR___rarg(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__29() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__28; +x_3 = l_List_appendTR___rarg(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__30() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_elabModuleDoc___closed__3; +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__29; +x_3 = l_List_foldl___at_String_join___spec__1(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__31() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__30; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__32() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__28; +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__13; +x_3 = l_List_appendTR___rarg(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__33() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_elabModuleDoc___closed__3; +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__32; +x_3 = l_List_foldl___at_String_join___spec__1(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__34() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__33; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__35() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__27; +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__18; +x_3 = l_List_appendTR___rarg(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__36() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__35; +x_3 = l_List_appendTR___rarg(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__37() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_elabModuleDoc___closed__3; +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__36; +x_3 = l_List_foldl___at_String_join___spec__1(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__38() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__37; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__39() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__35; +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__13; +x_3 = l_List_appendTR___rarg(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__40() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_elabModuleDoc___closed__3; +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__39; +x_3 = l_List_foldl___at_String_join___spec__1(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__41() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__40; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_6 = l_Lean_stringToMessageData(x_1); +x_7 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__7; +x_8 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_8, 0, x_7); +lean_ctor_set(x_8, 1, x_6); +x_9 = l_Lean_Elab_Command_elabModuleDoc___closed__4; +x_10 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_10, 0, x_8); +lean_ctor_set(x_10, 1, x_9); +x_11 = l_System_Platform_isWindows; +if (x_11 == 0) +{ +uint8_t x_12; +x_12 = l_System_Platform_isOSX; +if (x_12 == 0) +{ +uint8_t x_13; +x_13 = l_System_Platform_isEmscripten; +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; +x_14 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__11; +x_15 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_15, 0, x_10); +lean_ctor_set(x_15, 1, x_14); +x_16 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_16, 1, x_9); +x_17 = 0; +x_18 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_16, x_17, x_3, x_4, x_5); +return x_18; +} +else +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; +x_19 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__16; +x_20 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_20, 0, x_10); +lean_ctor_set(x_20, 1, x_19); +x_21 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_21, 0, x_20); +lean_ctor_set(x_21, 1, x_9); +x_22 = 0; +x_23 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_21, x_22, x_3, x_4, x_5); +return x_23; +} +} +else +{ +uint8_t x_24; +x_24 = l_System_Platform_isEmscripten; +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; lean_object* x_29; +x_25 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__22; +x_26 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_26, 0, x_10); +lean_ctor_set(x_26, 1, x_25); +x_27 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_9); +x_28 = 0; +x_29 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_27, x_28, x_3, x_4, x_5); +return x_29; +} +else +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; lean_object* x_34; +x_30 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__25; +x_31 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_31, 0, x_10); +lean_ctor_set(x_31, 1, x_30); +x_32 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_32, 0, x_31); +lean_ctor_set(x_32, 1, x_9); +x_33 = 0; +x_34 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_32, x_33, x_3, x_4, x_5); +return x_34; +} +} +} +else { -lean_object* x_5; uint8_t x_6; -x_5 = l_Lean_Elab_Command_elabOmit___closed__2; -lean_inc(x_1); -x_6 = l_Lean_Syntax_isOfKind(x_1, x_5); -if (x_6 == 0) +uint8_t x_35; +x_35 = l_System_Platform_isOSX; +if (x_35 == 0) { -lean_object* x_7; -lean_dec(x_1); -x_7 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabNamespace___spec__1___rarg(x_4); -return x_7; +uint8_t x_36; +x_36 = l_System_Platform_isEmscripten; +if (x_36 == 0) +{ +lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; lean_object* x_41; +x_37 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__31; +x_38 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_38, 0, x_10); +lean_ctor_set(x_38, 1, x_37); +x_39 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_39, 0, x_38); +lean_ctor_set(x_39, 1, x_9); +x_40 = 0; +x_41 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_39, x_40, x_3, x_4, x_5); +return x_41; } else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_8 = lean_unsigned_to_nat(1u); -x_9 = l_Lean_Syntax_getArg(x_1, x_8); -lean_dec(x_1); -x_10 = lean_box(0); -x_11 = l_Lean_Syntax_getArgs(x_9); -lean_dec(x_9); -x_12 = l_Lean_Elab_Command_elabSection___closed__4; -x_13 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___closed__2; -x_14 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabOmit___lambda__1___boxed), 12, 4); -lean_closure_set(x_14, 0, x_11); -lean_closure_set(x_14, 1, x_12); -lean_closure_set(x_14, 2, x_13); -lean_closure_set(x_14, 3, x_10); -x_15 = l_Lean_Elab_Command_runTermElabM___rarg(x_14, x_2, x_3, x_4); -if (lean_obj_tag(x_15) == 0) -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_16 = lean_ctor_get(x_15, 0); -lean_inc(x_16); -x_17 = lean_ctor_get(x_15, 1); -lean_inc(x_17); -lean_dec(x_15); -x_18 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabOmit___lambda__2), 3, 2); -lean_closure_set(x_18, 0, x_16); -lean_closure_set(x_18, 1, x_10); -x_19 = l_Lean_Elab_Command_modifyScope(x_18, x_2, x_3, x_17); -return x_19; +lean_object* x_42; lean_object* x_43; lean_object* x_44; uint8_t x_45; lean_object* x_46; +x_42 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__34; +x_43 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_43, 0, x_10); +lean_ctor_set(x_43, 1, x_42); +x_44 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_44, 0, x_43); +lean_ctor_set(x_44, 1, x_9); +x_45 = 0; +x_46 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_44, x_45, x_3, x_4, x_5); +return x_46; +} } else { -uint8_t x_20; -x_20 = !lean_is_exclusive(x_15); -if (x_20 == 0) +uint8_t x_47; +x_47 = l_System_Platform_isEmscripten; +if (x_47 == 0) { -return x_15; +lean_object* x_48; lean_object* x_49; lean_object* x_50; uint8_t x_51; lean_object* x_52; +x_48 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__38; +x_49 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_49, 0, x_10); +lean_ctor_set(x_49, 1, x_48); +x_50 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_50, 0, x_49); +lean_ctor_set(x_50, 1, x_9); +x_51 = 0; +x_52 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_50, x_51, x_3, x_4, x_5); +return x_52; } else { -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_15, 0); -x_22 = lean_ctor_get(x_15, 1); -lean_inc(x_22); -lean_inc(x_21); -lean_dec(x_15); -x_23 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_23, 0, x_21); -lean_ctor_set(x_23, 1, x_22); -return x_23; +lean_object* x_53; lean_object* x_54; lean_object* x_55; uint8_t x_56; lean_object* x_57; +x_53 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__41; +x_54 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_54, 0, x_10); +lean_ctor_set(x_54, 1, x_53); +x_55 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_55, 0, x_54); +lean_ctor_set(x_55, 1, x_9); +x_56 = 0; +x_57 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_55, x_56, x_3, x_4, x_5); +return x_57; } } } } } -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabOmit___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___closed__1() { _start: { -lean_object* x_7; -x_7 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabOmit___spec__1(x_1, x_2, x_3, x_4, x_5, x_6); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_7; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___boxed), 5, 0); +return x_1; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabOmit___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___closed__2() { _start: { -size_t x_14; size_t x_15; lean_object* x_16; -x_14 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_15 = lean_unbox_usize(x_5); -lean_dec(x_5); -x_16 = l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabOmit___spec__3(x_1, x_2, x_3, x_14, x_15, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_16; +lean_object* x_1; lean_object* x_2; +x_1 = l_System_Platform_target; +x_2 = lean_string_utf8_byte_size(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabOmit___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +static uint8_t _init_l_Lean_Elab_Command_elabVersion___rarg___closed__3() { _start: { -size_t x_4; size_t x_5; lean_object* x_6; -x_4 = lean_unbox_usize(x_1); -lean_dec(x_1); -x_5 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_6 = l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabOmit___spec__4(x_4, x_5, x_3); -return x_6; +lean_object* x_1; lean_object* x_2; uint8_t x_3; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___closed__2; +x_2 = lean_unsigned_to_nat(0u); +x_3 = lean_nat_dec_eq(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Elab_Command_elabOmit___spec__5___boxed(lean_object* x_1, lean_object* x_2) { +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___closed__4() { _start: { -uint8_t x_3; lean_object* x_4; -x_3 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Elab_Command_elabOmit___spec__5(x_1, x_2); -lean_dec(x_2); -lean_dec(x_1); -x_4 = lean_box(x_3); -return x_4; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("unknown", 7, 7); +return x_1; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Elab_Command_elabOmit___spec__10___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabVersion___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_3; -x_3 = l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Elab_Command_elabOmit___spec__10(x_1, x_2); -lean_dec(x_2); -lean_dec(x_1); -return x_3; -} +lean_object* x_4; uint8_t x_5; +x_4 = l_Lean_Elab_Command_elabVersion___rarg___closed__1; +x_5 = l_Lean_Elab_Command_elabVersion___rarg___closed__3; +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_6 = l_System_Platform_target; +x_7 = lean_box(0); +x_8 = lean_apply_5(x_4, x_6, x_7, x_1, x_2, x_3); +return x_8; } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__11___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: +else { -lean_object* x_11; -x_11 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__11___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = l_Lean_Elab_Command_elabVersion___rarg___closed__4; +x_10 = lean_box(0); +x_11 = lean_apply_5(x_4, x_9, x_10, x_1, x_2, x_3); return x_11; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { -_start: -{ -size_t x_14; size_t x_15; lean_object* x_16; -x_14 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_15 = lean_unbox_usize(x_5); -lean_dec(x_5); -x_16 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__11(x_1, x_2, x_3, x_14, x_15, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_1); -return x_16; -} } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__12___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabVersion(lean_object* x_1) { _start: { -lean_object* x_10; -x_10 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__12___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_10; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabVersion___rarg), 3, 0); +return x_2; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__12___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -size_t x_15; size_t x_16; size_t x_17; lean_object* x_18; -x_15 = lean_unbox_usize(x_1); -lean_dec(x_1); -x_16 = lean_unbox_usize(x_5); -lean_dec(x_5); -x_17 = lean_unbox_usize(x_6); -lean_dec(x_6); -x_18 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__12(x_15, x_2, x_3, x_4, x_16, x_17, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -lean_dec(x_9); +lean_object* x_6; +x_6 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5); lean_dec(x_4); lean_dec(x_2); -return x_18; -} -} -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -size_t x_12; size_t x_13; lean_object* x_14; -x_12 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_13 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_14 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__13(x_1, x_12, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); lean_dec(x_1); -return x_14; -} -} -LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at_Lean_Elab_Command_elabOmit___spec__14___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; -x_11 = l_Lean_RBNode_forIn_visit___at_Lean_Elab_Command_elabOmit___spec__14(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -return x_11; +return x_6; } } -LEAN_EXPORT lean_object* l_List_filterTR_loop___at_Lean_Elab_Command_elabOmit___spec__15___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabVersion___boxed(lean_object* x_1) { _start: { -lean_object* x_4; -x_4 = l_List_filterTR_loop___at_Lean_Elab_Command_elabOmit___spec__15(x_1, x_2, x_3); +lean_object* x_2; +x_2 = l_Lean_Elab_Command_elabVersion(x_1); lean_dec(x_1); -return x_4; +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabOmit___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__1() { _start: { -lean_object* x_13; -x_13 = l_Lean_Elab_Command_elabOmit___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_5); -lean_dec(x_3); -lean_dec(x_2); -return x_13; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("version", 7, 7); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabOmit___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__2() { _start: { -lean_object* x_5; -x_5 = l_Lean_Elab_Command_elabOmit(x_1, x_2, x_3, x_4); -lean_dec(x_3); -lean_dec(x_2); +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l___regBuiltin_Lean_Elab_Command_elabModuleDoc__1___closed__1; +x_2 = l___regBuiltin_Lean_Elab_Command_elabModuleDoc__1___closed__2; +x_3 = l___regBuiltin_Lean_Elab_Command_elabModuleDoc__1___closed__3; +x_4 = l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__1; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabOmit__1___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__3() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("elabOmit", 8, 8); +x_1 = lean_mk_string_unchecked("elabVersion", 11, 11); return x_1; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabOmit__1___closed__2() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l___regBuiltin_Lean_Elab_Command_elabModuleDoc__1___closed__1; x_2 = l___regBuiltin_Lean_Elab_Command_elabModuleDoc__1___closed__6; x_3 = l___regBuiltin_Lean_Elab_Command_elabModuleDoc__1___closed__3; -x_4 = l___regBuiltin_Lean_Elab_Command_elabOmit__1___closed__1; +x_4 = l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__3; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabOmit__1___closed__3() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__5() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabOmit___boxed), 4, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabVersion___boxed), 1, 0); return x_1; } } -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabOmit__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabVersion__1(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_2 = l___regBuiltin_Lean_Elab_Command_elabModuleDoc__1___closed__9; -x_3 = l_Lean_Elab_Command_elabOmit___closed__2; -x_4 = l___regBuiltin_Lean_Elab_Command_elabOmit__1___closed__2; -x_5 = l___regBuiltin_Lean_Elab_Command_elabOmit__1___closed__3; +x_3 = l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__2; +x_4 = l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__4; +x_5 = l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__5; x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); return x_6; } @@ -30226,6 +31740,7 @@ lean_object* initialize_Lean_Elab_Eval(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Elab_Command(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Elab_Open(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Elab_SetOption(uint8_t builtin, lean_object*); +lean_object* initialize_Init_System_Platform(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Lean_Elab_BuiltinCommand(uint8_t builtin, lean_object* w) { lean_object * res; @@ -30255,6 +31770,9 @@ lean_dec_ref(res); res = initialize_Lean_Elab_SetOption(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +res = initialize_Init_System_Platform(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Elab_Command_elabModuleDoc___closed__1 = _init_l_Lean_Elab_Command_elabModuleDoc___closed__1(); lean_mark_persistent(l_Lean_Elab_Command_elabModuleDoc___closed__1); l_Lean_Elab_Command_elabModuleDoc___closed__2 = _init_l_Lean_Elab_Command_elabModuleDoc___closed__2(); @@ -30561,12 +32079,12 @@ lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_elabInitQuot_declRange__1_ if (builtin) {res = l___regBuiltin_Lean_Elab_Command_elabInitQuot_declRange__1(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__1 = _init_l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__1(); -lean_mark_persistent(l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__1); -l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__2 = _init_l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__2(); -lean_mark_persistent(l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__2); -l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__3 = _init_l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__3(); -lean_mark_persistent(l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__3); +}l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__1 = _init_l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__1(); +lean_mark_persistent(l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__1); +l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__2 = _init_l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__2(); +lean_mark_persistent(l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__2); +l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__3 = _init_l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__3(); +lean_mark_persistent(l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__4___closed__3); l_Lean_resolveNamespace___at_Lean_Elab_Command_elabExport___spec__1___closed__1 = _init_l_Lean_resolveNamespace___at_Lean_Elab_Command_elabExport___spec__1___closed__1(); lean_mark_persistent(l_Lean_resolveNamespace___at_Lean_Elab_Command_elabExport___spec__1___closed__1); l_Lean_resolveNamespace___at_Lean_Elab_Command_elabExport___spec__1___closed__2 = _init_l_Lean_resolveNamespace___at_Lean_Elab_Command_elabExport___spec__1___closed__2(); @@ -30575,40 +32093,40 @@ l_Lean_resolveNamespace___at_Lean_Elab_Command_elabExport___spec__1___closed__3 lean_mark_persistent(l_Lean_resolveNamespace___at_Lean_Elab_Command_elabExport___spec__1___closed__3); l_Lean_resolveNamespace___at_Lean_Elab_Command_elabExport___spec__1___closed__4 = _init_l_Lean_resolveNamespace___at_Lean_Elab_Command_elabExport___spec__1___closed__4(); lean_mark_persistent(l_Lean_resolveNamespace___at_Lean_Elab_Command_elabExport___spec__1___closed__4); -l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__11___closed__1 = _init_l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__11___closed__1(); -lean_mark_persistent(l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__11___closed__1); -l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__11___closed__2 = _init_l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__11___closed__2(); -lean_mark_persistent(l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__11___closed__2); -l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__11___closed__3 = _init_l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__11___closed__3(); -lean_mark_persistent(l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__11___closed__3); -l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__13___closed__1 = _init_l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__13___closed__1(); -lean_mark_persistent(l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__13___closed__1); -l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__13___closed__2 = _init_l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__13___closed__2(); -lean_mark_persistent(l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__13___closed__2); -l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__1 = _init_l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__1(); -lean_mark_persistent(l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__1); -l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__2 = _init_l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__2(); -lean_mark_persistent(l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__2); -l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__3 = _init_l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__3(); -lean_mark_persistent(l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__3); -l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__4 = _init_l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__4(); -lean_mark_persistent(l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__19___closed__4); -l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__18___closed__1 = _init_l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__18___closed__1(); -lean_mark_persistent(l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__18___closed__1); -l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__18___closed__2 = _init_l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__18___closed__2(); -lean_mark_persistent(l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__18___closed__2); -l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___lambda__1___closed__1 = _init_l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___lambda__1___closed__1(); -lean_mark_persistent(l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___lambda__1___closed__1); -l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___lambda__1___closed__2 = _init_l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___lambda__1___closed__2(); -lean_mark_persistent(l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___lambda__1___closed__2); -l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___closed__1 = _init_l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___closed__1(); -lean_mark_persistent(l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___closed__1); -l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___closed__2 = _init_l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___closed__2(); -lean_mark_persistent(l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___closed__2); -l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___closed__3 = _init_l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___closed__3(); -lean_mark_persistent(l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___closed__3); -l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___closed__4 = _init_l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___closed__4(); -lean_mark_persistent(l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___closed__4); +l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__12___closed__1 = _init_l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__12___closed__1(); +lean_mark_persistent(l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__12___closed__1); +l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__12___closed__2 = _init_l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__12___closed__2(); +lean_mark_persistent(l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__12___closed__2); +l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__12___closed__3 = _init_l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__12___closed__3(); +lean_mark_persistent(l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__12___closed__3); +l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__14___closed__1 = _init_l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__14___closed__1(); +lean_mark_persistent(l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__14___closed__1); +l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__14___closed__2 = _init_l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__14___closed__2(); +lean_mark_persistent(l_Lean_ensureNoOverload___at_Lean_Elab_Command_elabExport___spec__14___closed__2); +l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__1 = _init_l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__1(); +lean_mark_persistent(l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__1); +l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__2 = _init_l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__2(); +lean_mark_persistent(l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__2); +l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__3 = _init_l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__3(); +lean_mark_persistent(l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__3); +l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__4 = _init_l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__4(); +lean_mark_persistent(l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Command_elabExport___spec__20___closed__4); +l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__19___closed__1 = _init_l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__19___closed__1(); +lean_mark_persistent(l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__19___closed__1); +l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__19___closed__2 = _init_l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__19___closed__2(); +lean_mark_persistent(l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__19___closed__2); +l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___lambda__1___closed__1 = _init_l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___lambda__1___closed__1(); +lean_mark_persistent(l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___lambda__1___closed__1); +l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___lambda__1___closed__2 = _init_l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___lambda__1___closed__2(); +lean_mark_persistent(l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___lambda__1___closed__2); +l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___closed__1 = _init_l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___closed__1(); +lean_mark_persistent(l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___closed__1); +l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___closed__2 = _init_l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___closed__2(); +lean_mark_persistent(l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___closed__2); +l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___closed__3 = _init_l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___closed__3(); +lean_mark_persistent(l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___closed__3); +l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___closed__4 = _init_l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___closed__4(); +lean_mark_persistent(l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__6___closed__4); l_Lean_Elab_Command_elabExport___closed__1 = _init_l_Lean_Elab_Command_elabExport___closed__1(); lean_mark_persistent(l_Lean_Elab_Command_elabExport___closed__1); l_Lean_Elab_Command_elabExport___closed__2 = _init_l_Lean_Elab_Command_elabExport___closed__2(); @@ -30727,22 +32245,10 @@ l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_typelessBinder_x3f___c lean_mark_persistent(l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_typelessBinder_x3f___closed__4); l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_typelessBinder_x3f___closed__5 = _init_l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_typelessBinder_x3f___closed__5(); lean_mark_persistent(l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_typelessBinder_x3f___closed__5); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__2___closed__1 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__2___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__2___closed__1); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__2___closed__2 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__2___closed__2(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__2___closed__2); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__1 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__1); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__2 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__2(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__2); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__3 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__3(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__3); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__4 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__4(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__4); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__5 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__5(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__5); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__6 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__6(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__6); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__3___closed__1 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__3___closed__1(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__3___closed__1); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__3___closed__2 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__3___closed__2(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__3___closed__2); l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__1 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__1(); lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__1); l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__2 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__2(); @@ -30751,16 +32257,28 @@ l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Co lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__3); l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__4 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__4(); lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__4); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__5 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__5(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__5); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__6 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__6(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__6); l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6___closed__1 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6___closed__1(); lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6___closed__1); l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6___closed__2 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6___closed__2(); lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6___closed__2); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6___closed__3 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6___closed__3(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6___closed__3); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6___closed__4 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6___closed__4(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6___closed__4); l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___closed__1 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___closed__1(); lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___closed__1); l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___closed__2 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___closed__2(); lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___closed__2); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___closed__3 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___closed__3(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___closed__3); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___closed__1 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___closed__1(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___closed__1); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___closed__2 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___closed__2(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___closed__2); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___closed__3 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___closed__3(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__8___closed__3); l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___closed__1 = _init_l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___closed__1(); lean_mark_persistent(l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___closed__1); l_Lean_Elab_Command_elabVariable___lambda__2___closed__1 = _init_l_Lean_Elab_Command_elabVariable___lambda__2___closed__1(); @@ -31025,6 +32543,12 @@ l_Lean_getDocStringText___at_Lean_Elab_Command_elabAddDeclDoc___spec__2___closed lean_mark_persistent(l_Lean_getDocStringText___at_Lean_Elab_Command_elabAddDeclDoc___spec__2___closed__1); l_Lean_getDocStringText___at_Lean_Elab_Command_elabAddDeclDoc___spec__2___closed__2 = _init_l_Lean_getDocStringText___at_Lean_Elab_Command_elabAddDeclDoc___spec__2___closed__2(); lean_mark_persistent(l_Lean_getDocStringText___at_Lean_Elab_Command_elabAddDeclDoc___spec__2___closed__2); +l_Lean_addDocString___at_Lean_Elab_Command_elabAddDeclDoc___spec__5___lambda__1___closed__1 = _init_l_Lean_addDocString___at_Lean_Elab_Command_elabAddDeclDoc___spec__5___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_addDocString___at_Lean_Elab_Command_elabAddDeclDoc___spec__5___lambda__1___closed__1); +l_Lean_addDocString___at_Lean_Elab_Command_elabAddDeclDoc___spec__5___closed__1 = _init_l_Lean_addDocString___at_Lean_Elab_Command_elabAddDeclDoc___spec__5___closed__1(); +lean_mark_persistent(l_Lean_addDocString___at_Lean_Elab_Command_elabAddDeclDoc___spec__5___closed__1); +l_Lean_addDocString___at_Lean_Elab_Command_elabAddDeclDoc___spec__5___closed__2 = _init_l_Lean_addDocString___at_Lean_Elab_Command_elabAddDeclDoc___spec__5___closed__2(); +lean_mark_persistent(l_Lean_addDocString___at_Lean_Elab_Command_elabAddDeclDoc___spec__5___closed__2); l_Lean_Elab_Command_elabAddDeclDoc___closed__1 = _init_l_Lean_Elab_Command_elabAddDeclDoc___closed__1(); lean_mark_persistent(l_Lean_Elab_Command_elabAddDeclDoc___closed__1); l_Lean_Elab_Command_elabAddDeclDoc___closed__2 = _init_l_Lean_Elab_Command_elabAddDeclDoc___closed__2(); @@ -31113,6 +32637,108 @@ lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_elabOmit__1___closed__3); if (builtin) {res = l___regBuiltin_Lean_Elab_Command_elabOmit__1(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +}l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__1 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__1); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__2 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__2); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__3 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__3); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__4 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__4); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__5 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__5); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__6 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__6); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__7 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__7(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__7); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__8 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__8(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__8); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__9 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__9(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__9); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__10 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__10(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__10); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__11 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__11(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__11); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__12 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__12(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__12); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__13 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__13(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__13); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__14 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__14(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__14); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__15 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__15(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__15); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__16 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__16(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__16); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__17 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__17(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__17); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__18 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__18(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__18); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__19 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__19(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__19); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__20 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__20(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__20); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__21 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__21(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__21); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__22 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__22(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__22); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__23 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__23(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__23); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__24 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__24(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__24); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__25 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__25(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__25); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__26 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__26(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__26); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__27 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__27(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__27); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__28 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__28(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__28); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__29 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__29(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__29); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__30 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__30(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__30); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__31 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__31(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__31); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__32 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__32(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__32); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__33 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__33(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__33); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__34 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__34(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__34); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__35 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__35(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__35); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__36 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__36(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__36); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__37 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__37(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__37); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__38 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__38(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__38); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__39 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__39(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__39); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__40 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__40(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__40); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__41 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__41(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__41); +l_Lean_Elab_Command_elabVersion___rarg___closed__1 = _init_l_Lean_Elab_Command_elabVersion___rarg___closed__1(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___closed__1); +l_Lean_Elab_Command_elabVersion___rarg___closed__2 = _init_l_Lean_Elab_Command_elabVersion___rarg___closed__2(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___closed__2); +l_Lean_Elab_Command_elabVersion___rarg___closed__3 = _init_l_Lean_Elab_Command_elabVersion___rarg___closed__3(); +l_Lean_Elab_Command_elabVersion___rarg___closed__4 = _init_l_Lean_Elab_Command_elabVersion___rarg___closed__4(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___closed__4); +l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__1 = _init_l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__1); +l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__2 = _init_l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__2); +l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__3 = _init_l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__3); +l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__4 = _init_l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__4(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__4); +l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__5 = _init_l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__5(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__5); +if (builtin) {res = l___regBuiltin_Lean_Elab_Command_elabVersion__1(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); }l_Lean_logWarning___at_Lean_Elab_Command_elabExit___spec__1___closed__1 = _init_l_Lean_logWarning___at_Lean_Elab_Command_elabExit___spec__1___closed__1(); lean_mark_persistent(l_Lean_logWarning___at_Lean_Elab_Command_elabExit___spec__1___closed__1); l_Lean_Elab_Command_elabExit___rarg___closed__1 = _init_l_Lean_Elab_Command_elabExit___rarg___closed__1(); diff --git a/stage0/stdlib/Lean/Elab/BuiltinEvalCommand.c b/stage0/stdlib/Lean/Elab/BuiltinEvalCommand.c index fc9cd3ce4e5d..d3e31c3ab526 100644 --- a/stage0/stdlib/Lean/Elab/BuiltinEvalCommand.c +++ b/stage0/stdlib/Lean/Elab/BuiltinEvalCommand.c @@ -240,7 +240,7 @@ lean_object* l_Lean_Meta_mkAppM(lean_object*, lean_object*, lean_object*, lean_o static lean_object* l_Lean_Elab_Command_elabRunCmd___lambda__1___closed__7; static lean_object* l_Lean_Elab_Command_elabEvalCoreUnsafe___lambda__17___closed__40; lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_liftCommandElabM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_liftCommandElabM___rarg(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabRunCmd___lambda__1___closed__11; static lean_object* l___private_Lean_Elab_BuiltinEvalCommand_0__Lean_Elab_Command_addAndCompileExprForEval___closed__27; lean_object* lean_st_mk_ref(lean_object*, lean_object*); @@ -324,7 +324,6 @@ static lean_object* l___regBuiltin_Lean_Elab_Command_elabRunElab_declRange__1___ LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabEvalCoreUnsafe___lambda__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofConstName(lean_object*); static lean_object* l___private_Lean_Elab_BuiltinEvalCommand_0__Lean_Elab_Command_addAndCompileExprForEval___closed__4; -lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Environment_contains(lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofExpr(lean_object*); lean_object* l_Lean_Option_register___at_Lean_Elab_initFn____x40_Lean_Elab_AutoBound___hyg_6____spec__1(lean_object*, lean_object*, lean_object*, lean_object*); @@ -473,6 +472,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_BuiltinEval uint8_t lean_usize_dec_lt(size_t, size_t); static lean_object* l___regBuiltin_Lean_Elab_Command_elabRunElab__1___closed__3; static lean_object* l___private_Lean_Elab_BuiltinEvalCommand_0__Lean_Elab_Command_mkFormat___closed__3; +lean_object* l_Lean_throwError___at_Lean_withSetOptionIn___spec__7(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkLambdaFVars(lean_object*, lean_object*, uint8_t, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabEvalCoreUnsafe___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_BuiltinEvalCommand_0__Lean_Elab_Command_mkFormat___lambda__1___closed__2; @@ -2985,21 +2985,23 @@ return x_5; static lean_object* _init_l___private_Lean_Elab_BuiltinEvalCommand_0__Lean_Elab_Command_addAndCompileExprForEval___closed__22() { _start: { -lean_object* x_1; uint8_t x_2; uint8_t x_3; uint8_t x_4; uint8_t x_5; lean_object* x_6; lean_object* x_7; +lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; uint8_t x_5; uint8_t x_6; lean_object* x_7; lean_object* x_8; x_1 = lean_box(0); -x_2 = 0; +x_2 = lean_box(0); x_3 = 0; -x_4 = 2; -x_5 = 1; -x_6 = l_Lean_collectAxioms___at___private_Lean_Elab_BuiltinEvalCommand_0__Lean_Elab_Command_addAndCompileExprForEval___spec__1___closed__1; -x_7 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_7, 0, x_1); -lean_ctor_set(x_7, 1, x_6); -lean_ctor_set_uint8(x_7, sizeof(void*)*2, x_2); -lean_ctor_set_uint8(x_7, sizeof(void*)*2 + 1, x_3); -lean_ctor_set_uint8(x_7, sizeof(void*)*2 + 2, x_4); -lean_ctor_set_uint8(x_7, sizeof(void*)*2 + 3, x_5); -return x_7; +x_4 = 0; +x_5 = 2; +x_6 = 1; +x_7 = l_Lean_collectAxioms___at___private_Lean_Elab_BuiltinEvalCommand_0__Lean_Elab_Command_addAndCompileExprForEval___spec__1___closed__1; +x_8 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_8, 0, x_2); +lean_ctor_set(x_8, 1, x_1); +lean_ctor_set(x_8, 2, x_7); +lean_ctor_set_uint8(x_8, sizeof(void*)*3, x_3); +lean_ctor_set_uint8(x_8, sizeof(void*)*3 + 1, x_4); +lean_ctor_set_uint8(x_8, sizeof(void*)*3 + 2, x_5); +lean_ctor_set_uint8(x_8, sizeof(void*)*3 + 3, x_6); +return x_8; } } static lean_object* _init_l___private_Lean_Elab_BuiltinEvalCommand_0__Lean_Elab_Command_addAndCompileExprForEval___closed__23() { @@ -4498,7 +4500,7 @@ return x_2; LEAN_EXPORT lean_object* l___private_Lean_Elab_BuiltinEvalCommand_0__Lean_Elab_Command_mkFormat___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +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; x_10 = lean_box(0); x_11 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_11, 0, x_1); @@ -4510,314 +4512,315 @@ x_14 = lean_alloc_closure((void*)(l_Lean_Elab_applyDerivingHandlers), 6, 3); lean_closure_set(x_14, 0, x_13); lean_closure_set(x_14, 1, x_12); lean_closure_set(x_14, 2, x_2); -x_15 = l_Lean_liftCommandElabM___rarg(x_14, x_7, x_8, x_9); -if (lean_obj_tag(x_15) == 0) +x_15 = 1; +x_16 = l_Lean_liftCommandElabM___rarg(x_14, x_15, x_7, x_8, x_9); +if (lean_obj_tag(x_16) == 0) { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; -x_16 = lean_ctor_get(x_15, 1); -lean_inc(x_16); -lean_dec(x_15); -x_17 = lean_st_ref_take(x_6, x_16); -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_17, 1); +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_17 = lean_ctor_get(x_16, 1); +lean_inc(x_17); +lean_dec(x_16); +x_18 = lean_st_ref_take(x_6, x_17); +x_19 = lean_ctor_get(x_18, 0); lean_inc(x_19); -lean_dec(x_17); -x_20 = !lean_is_exclusive(x_18); -if (x_20 == 0) +x_20 = lean_ctor_get(x_18, 1); +lean_inc(x_20); +lean_dec(x_18); +x_21 = !lean_is_exclusive(x_19); +if (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; 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_18, 1); -x_22 = lean_ctor_get(x_21, 0); -lean_inc(x_22); -x_23 = lean_ctor_get(x_21, 1); +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_19, 1); +x_23 = lean_ctor_get(x_22, 0); lean_inc(x_23); -x_24 = lean_ctor_get(x_21, 3); +x_24 = lean_ctor_get(x_22, 1); lean_inc(x_24); -x_25 = lean_ctor_get(x_21, 4); +x_25 = lean_ctor_get(x_22, 3); lean_inc(x_25); -x_26 = lean_ctor_get(x_21, 5); +x_26 = lean_ctor_get(x_22, 4); lean_inc(x_26); -x_27 = lean_ctor_get(x_21, 6); +x_27 = lean_ctor_get(x_22, 5); lean_inc(x_27); -lean_dec(x_21); -x_28 = l___private_Lean_Elab_BuiltinEvalCommand_0__Lean_Elab_Command_mkFormat___lambda__2___closed__2; -x_29 = lean_alloc_ctor(0, 7, 0); -lean_ctor_set(x_29, 0, x_22); -lean_ctor_set(x_29, 1, x_23); -lean_ctor_set(x_29, 2, x_28); -lean_ctor_set(x_29, 3, x_24); -lean_ctor_set(x_29, 4, x_25); -lean_ctor_set(x_29, 5, x_26); -lean_ctor_set(x_29, 6, x_27); -lean_ctor_set(x_18, 1, x_29); -x_30 = lean_st_ref_set(x_6, x_18, x_19); -x_31 = !lean_is_exclusive(x_30); -if (x_31 == 0) +x_28 = lean_ctor_get(x_22, 6); +lean_inc(x_28); +lean_dec(x_22); +x_29 = l___private_Lean_Elab_BuiltinEvalCommand_0__Lean_Elab_Command_mkFormat___lambda__2___closed__2; +x_30 = lean_alloc_ctor(0, 7, 0); +lean_ctor_set(x_30, 0, x_23); +lean_ctor_set(x_30, 1, x_24); +lean_ctor_set(x_30, 2, x_29); +lean_ctor_set(x_30, 3, x_25); +lean_ctor_set(x_30, 4, x_26); +lean_ctor_set(x_30, 5, x_27); +lean_ctor_set(x_30, 6, x_28); +lean_ctor_set(x_19, 1, x_30); +x_31 = lean_st_ref_set(x_6, x_19, x_20); +x_32 = !lean_is_exclusive(x_31); +if (x_32 == 0) { -lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_32 = lean_ctor_get(x_30, 1); -x_33 = lean_ctor_get(x_30, 0); -lean_dec(x_33); -x_34 = l___private_Lean_Elab_BuiltinEvalCommand_0__Lean_Elab_Command_mkRepr(x_3, x_2, x_5, x_6, x_7, x_8, x_32); -if (lean_obj_tag(x_34) == 0) +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_31, 1); +x_34 = lean_ctor_get(x_31, 0); +lean_dec(x_34); +x_35 = l___private_Lean_Elab_BuiltinEvalCommand_0__Lean_Elab_Command_mkRepr(x_3, x_2, x_5, x_6, x_7, x_8, x_33); +if (lean_obj_tag(x_35) == 0) { -uint8_t x_35; -x_35 = !lean_is_exclusive(x_34); -if (x_35 == 0) +uint8_t x_36; +x_36 = !lean_is_exclusive(x_35); +if (x_36 == 0) { -lean_object* x_36; lean_object* x_37; -x_36 = lean_ctor_get(x_34, 0); -x_37 = lean_box(0); -lean_ctor_set_tag(x_30, 1); -lean_ctor_set(x_30, 1, x_37); -lean_ctor_set(x_30, 0, x_36); -lean_ctor_set(x_34, 0, x_30); -return x_34; +lean_object* x_37; lean_object* x_38; +x_37 = lean_ctor_get(x_35, 0); +x_38 = lean_box(0); +lean_ctor_set_tag(x_31, 1); +lean_ctor_set(x_31, 1, x_38); +lean_ctor_set(x_31, 0, x_37); +lean_ctor_set(x_35, 0, x_31); +return x_35; } 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_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; +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_inc(x_38); -lean_dec(x_34); -x_40 = lean_box(0); -lean_ctor_set_tag(x_30, 1); -lean_ctor_set(x_30, 1, x_40); -lean_ctor_set(x_30, 0, x_38); -x_41 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_41, 0, x_30); -lean_ctor_set(x_41, 1, x_39); -return x_41; +lean_dec(x_35); +x_41 = lean_box(0); +lean_ctor_set_tag(x_31, 1); +lean_ctor_set(x_31, 1, x_41); +lean_ctor_set(x_31, 0, x_39); +x_42 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_42, 0, x_31); +lean_ctor_set(x_42, 1, x_40); +return x_42; } } else { -uint8_t x_42; -lean_free_object(x_30); -x_42 = !lean_is_exclusive(x_34); -if (x_42 == 0) +uint8_t x_43; +lean_free_object(x_31); +x_43 = !lean_is_exclusive(x_35); +if (x_43 == 0) { -return x_34; +return x_35; } else { -lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_43 = lean_ctor_get(x_34, 0); -x_44 = lean_ctor_get(x_34, 1); +lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_44 = lean_ctor_get(x_35, 0); +x_45 = lean_ctor_get(x_35, 1); +lean_inc(x_45); lean_inc(x_44); -lean_inc(x_43); -lean_dec(x_34); -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_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; } } } else { -lean_object* x_46; lean_object* x_47; -x_46 = lean_ctor_get(x_30, 1); -lean_inc(x_46); -lean_dec(x_30); -x_47 = l___private_Lean_Elab_BuiltinEvalCommand_0__Lean_Elab_Command_mkRepr(x_3, x_2, x_5, x_6, x_7, x_8, x_46); -if (lean_obj_tag(x_47) == 0) +lean_object* x_47; lean_object* x_48; +x_47 = lean_ctor_get(x_31, 1); +lean_inc(x_47); +lean_dec(x_31); +x_48 = l___private_Lean_Elab_BuiltinEvalCommand_0__Lean_Elab_Command_mkRepr(x_3, x_2, x_5, x_6, x_7, x_8, x_47); +if (lean_obj_tag(x_48) == 0) { -lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; -x_48 = lean_ctor_get(x_47, 0); -lean_inc(x_48); -x_49 = lean_ctor_get(x_47, 1); +lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_49 = lean_ctor_get(x_48, 0); lean_inc(x_49); -if (lean_is_exclusive(x_47)) { - lean_ctor_release(x_47, 0); - lean_ctor_release(x_47, 1); - x_50 = x_47; +x_50 = lean_ctor_get(x_48, 1); +lean_inc(x_50); +if (lean_is_exclusive(x_48)) { + lean_ctor_release(x_48, 0); + lean_ctor_release(x_48, 1); + x_51 = x_48; } else { - lean_dec_ref(x_47); - x_50 = lean_box(0); + lean_dec_ref(x_48); + x_51 = lean_box(0); } -x_51 = lean_box(0); -x_52 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_52, 0, x_48); -lean_ctor_set(x_52, 1, x_51); -if (lean_is_scalar(x_50)) { - x_53 = lean_alloc_ctor(0, 2, 0); +x_52 = lean_box(0); +x_53 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_53, 0, x_49); +lean_ctor_set(x_53, 1, x_52); +if (lean_is_scalar(x_51)) { + x_54 = lean_alloc_ctor(0, 2, 0); } else { - x_53 = x_50; + x_54 = x_51; } -lean_ctor_set(x_53, 0, x_52); -lean_ctor_set(x_53, 1, x_49); -return x_53; +lean_ctor_set(x_54, 0, x_53); +lean_ctor_set(x_54, 1, x_50); +return x_54; } else { -lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; -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; lean_object* x_57; lean_object* x_58; +x_55 = lean_ctor_get(x_48, 0); lean_inc(x_55); -if (lean_is_exclusive(x_47)) { - lean_ctor_release(x_47, 0); - lean_ctor_release(x_47, 1); - x_56 = x_47; +x_56 = lean_ctor_get(x_48, 1); +lean_inc(x_56); +if (lean_is_exclusive(x_48)) { + lean_ctor_release(x_48, 0); + lean_ctor_release(x_48, 1); + x_57 = x_48; } else { - lean_dec_ref(x_47); - x_56 = lean_box(0); + lean_dec_ref(x_48); + x_57 = lean_box(0); } -if (lean_is_scalar(x_56)) { - x_57 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_57)) { + x_58 = lean_alloc_ctor(1, 2, 0); } else { - x_57 = x_56; + x_58 = x_57; } -lean_ctor_set(x_57, 0, x_54); -lean_ctor_set(x_57, 1, x_55); -return x_57; +lean_ctor_set(x_58, 0, x_55); +lean_ctor_set(x_58, 1, x_56); +return x_58; } } } else { -lean_object* x_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_58 = lean_ctor_get(x_18, 0); -x_59 = lean_ctor_get(x_18, 1); -x_60 = lean_ctor_get(x_18, 2); -x_61 = lean_ctor_get(x_18, 3); -x_62 = lean_ctor_get(x_18, 4); +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_59 = lean_ctor_get(x_19, 0); +x_60 = lean_ctor_get(x_19, 1); +x_61 = lean_ctor_get(x_19, 2); +x_62 = lean_ctor_get(x_19, 3); +x_63 = lean_ctor_get(x_19, 4); +lean_inc(x_63); lean_inc(x_62); lean_inc(x_61); lean_inc(x_60); lean_inc(x_59); -lean_inc(x_58); -lean_dec(x_18); -x_63 = lean_ctor_get(x_59, 0); -lean_inc(x_63); -x_64 = lean_ctor_get(x_59, 1); +lean_dec(x_19); +x_64 = lean_ctor_get(x_60, 0); lean_inc(x_64); -x_65 = lean_ctor_get(x_59, 3); +x_65 = lean_ctor_get(x_60, 1); lean_inc(x_65); -x_66 = lean_ctor_get(x_59, 4); +x_66 = lean_ctor_get(x_60, 3); lean_inc(x_66); -x_67 = lean_ctor_get(x_59, 5); +x_67 = lean_ctor_get(x_60, 4); lean_inc(x_67); -x_68 = lean_ctor_get(x_59, 6); +x_68 = lean_ctor_get(x_60, 5); lean_inc(x_68); -lean_dec(x_59); -x_69 = l___private_Lean_Elab_BuiltinEvalCommand_0__Lean_Elab_Command_mkFormat___lambda__2___closed__2; -x_70 = lean_alloc_ctor(0, 7, 0); -lean_ctor_set(x_70, 0, x_63); -lean_ctor_set(x_70, 1, x_64); -lean_ctor_set(x_70, 2, x_69); -lean_ctor_set(x_70, 3, x_65); -lean_ctor_set(x_70, 4, x_66); -lean_ctor_set(x_70, 5, x_67); -lean_ctor_set(x_70, 6, x_68); -x_71 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_71, 0, x_58); -lean_ctor_set(x_71, 1, x_70); -lean_ctor_set(x_71, 2, x_60); -lean_ctor_set(x_71, 3, x_61); -lean_ctor_set(x_71, 4, x_62); -x_72 = lean_st_ref_set(x_6, x_71, x_19); -x_73 = lean_ctor_get(x_72, 1); -lean_inc(x_73); -if (lean_is_exclusive(x_72)) { - lean_ctor_release(x_72, 0); - lean_ctor_release(x_72, 1); - x_74 = x_72; +x_69 = lean_ctor_get(x_60, 6); +lean_inc(x_69); +lean_dec(x_60); +x_70 = l___private_Lean_Elab_BuiltinEvalCommand_0__Lean_Elab_Command_mkFormat___lambda__2___closed__2; +x_71 = lean_alloc_ctor(0, 7, 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_66); +lean_ctor_set(x_71, 4, x_67); +lean_ctor_set(x_71, 5, x_68); +lean_ctor_set(x_71, 6, x_69); +x_72 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_72, 0, x_59); +lean_ctor_set(x_72, 1, x_71); +lean_ctor_set(x_72, 2, x_61); +lean_ctor_set(x_72, 3, x_62); +lean_ctor_set(x_72, 4, x_63); +x_73 = lean_st_ref_set(x_6, x_72, x_20); +x_74 = lean_ctor_get(x_73, 1); +lean_inc(x_74); +if (lean_is_exclusive(x_73)) { + lean_ctor_release(x_73, 0); + lean_ctor_release(x_73, 1); + x_75 = x_73; } else { - lean_dec_ref(x_72); - x_74 = lean_box(0); + lean_dec_ref(x_73); + x_75 = lean_box(0); } -x_75 = l___private_Lean_Elab_BuiltinEvalCommand_0__Lean_Elab_Command_mkRepr(x_3, x_2, x_5, x_6, x_7, x_8, x_73); -if (lean_obj_tag(x_75) == 0) +x_76 = l___private_Lean_Elab_BuiltinEvalCommand_0__Lean_Elab_Command_mkRepr(x_3, x_2, x_5, x_6, x_7, x_8, x_74); +if (lean_obj_tag(x_76) == 0) { -lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; -x_76 = lean_ctor_get(x_75, 0); -lean_inc(x_76); -x_77 = lean_ctor_get(x_75, 1); +lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; +x_77 = lean_ctor_get(x_76, 0); lean_inc(x_77); -if (lean_is_exclusive(x_75)) { - lean_ctor_release(x_75, 0); - lean_ctor_release(x_75, 1); - x_78 = x_75; +x_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_75); - x_78 = lean_box(0); + lean_dec_ref(x_76); + x_79 = lean_box(0); } -x_79 = lean_box(0); -if (lean_is_scalar(x_74)) { - x_80 = lean_alloc_ctor(1, 2, 0); +x_80 = lean_box(0); +if (lean_is_scalar(x_75)) { + x_81 = lean_alloc_ctor(1, 2, 0); } else { - x_80 = x_74; - lean_ctor_set_tag(x_80, 1); + x_81 = x_75; + lean_ctor_set_tag(x_81, 1); } -lean_ctor_set(x_80, 0, x_76); -lean_ctor_set(x_80, 1, x_79); -if (lean_is_scalar(x_78)) { - x_81 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_81, 0, x_77); +lean_ctor_set(x_81, 1, x_80); +if (lean_is_scalar(x_79)) { + x_82 = lean_alloc_ctor(0, 2, 0); } else { - x_81 = x_78; + x_82 = x_79; } -lean_ctor_set(x_81, 0, x_80); -lean_ctor_set(x_81, 1, x_77); -return x_81; +lean_ctor_set(x_82, 0, x_81); +lean_ctor_set(x_82, 1, x_78); +return x_82; } else { -lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; -lean_dec(x_74); -x_82 = lean_ctor_get(x_75, 0); -lean_inc(x_82); -x_83 = lean_ctor_get(x_75, 1); +lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; +lean_dec(x_75); +x_83 = lean_ctor_get(x_76, 0); lean_inc(x_83); -if (lean_is_exclusive(x_75)) { - lean_ctor_release(x_75, 0); - lean_ctor_release(x_75, 1); - x_84 = x_75; +x_84 = lean_ctor_get(x_76, 1); +lean_inc(x_84); +if (lean_is_exclusive(x_76)) { + lean_ctor_release(x_76, 0); + lean_ctor_release(x_76, 1); + x_85 = x_76; } else { - lean_dec_ref(x_75); - x_84 = lean_box(0); + lean_dec_ref(x_76); + x_85 = lean_box(0); } -if (lean_is_scalar(x_84)) { - x_85 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_85)) { + x_86 = lean_alloc_ctor(1, 2, 0); } else { - x_85 = x_84; + x_86 = x_85; } -lean_ctor_set(x_85, 0, x_82); -lean_ctor_set(x_85, 1, x_83); -return x_85; +lean_ctor_set(x_86, 0, x_83); +lean_ctor_set(x_86, 1, x_84); +return x_86; } } } else { -uint8_t x_86; +uint8_t x_87; 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_86 = !lean_is_exclusive(x_15); -if (x_86 == 0) +x_87 = !lean_is_exclusive(x_16); +if (x_87 == 0) { -return x_15; +return x_16; } else { -lean_object* x_87; lean_object* x_88; lean_object* x_89; -x_87 = lean_ctor_get(x_15, 0); -x_88 = lean_ctor_get(x_15, 1); +lean_object* x_88; lean_object* x_89; lean_object* x_90; +x_88 = lean_ctor_get(x_16, 0); +x_89 = lean_ctor_get(x_16, 1); +lean_inc(x_89); lean_inc(x_88); -lean_inc(x_87); -lean_dec(x_15); -x_89 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_89, 0, x_87); -lean_ctor_set(x_89, 1, x_88); -return x_89; +lean_dec(x_16); +x_90 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_90, 0, x_88); +lean_ctor_set(x_90, 1, x_89); +return x_90; } } } @@ -21148,7 +21151,7 @@ lean_object* x_18; lean_object* x_19; uint8_t x_20; lean_dec(x_11); lean_dec(x_9); x_18 = l_Lean_Elab_Command_elabRunCmd___closed__4; -x_19 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_18, x_2, x_3, x_14); +x_19 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__7(x_18, x_2, x_3, x_14); lean_dec(x_3); x_20 = !lean_is_exclusive(x_19); if (x_20 == 0) @@ -21518,7 +21521,7 @@ lean_object* x_18; lean_object* x_19; uint8_t x_20; lean_dec(x_11); lean_dec(x_9); x_18 = l_Lean_Elab_Command_elabRunElab___closed__4; -x_19 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_18, x_2, x_3, x_14); +x_19 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__7(x_18, x_2, x_3, x_14); lean_dec(x_3); x_20 = !lean_is_exclusive(x_19); if (x_20 == 0) @@ -21888,7 +21891,7 @@ lean_object* x_18; lean_object* x_19; uint8_t x_20; lean_dec(x_11); lean_dec(x_9); x_18 = l_Lean_Elab_Command_elabRunMeta___closed__4; -x_19 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_18, x_2, x_3, x_14); +x_19 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__7(x_18, x_2, x_3, x_14); lean_dec(x_3); x_20 = !lean_is_exclusive(x_19); if (x_20 == 0) diff --git a/stage0/stdlib/Lean/Elab/BuiltinNotation.c b/stage0/stdlib/Lean/Elab/BuiltinNotation.c index aaeb9122c31a..2854e2a845b5 100644 --- a/stage0/stdlib/Lean/Elab/BuiltinNotation.c +++ b/stage0/stdlib/Lean/Elab/BuiltinNotation.c @@ -422,6 +422,7 @@ static lean_object* l___regBuiltin_Lean_Elab_Term_elabBorrowed_declRange__1___cl lean_object* l_Lean_Meta_withLetDecl___at_Lean_Elab_Term_elabLetDeclAux___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_expr_eqv(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeReducing___at_Lean_Elab_Term_elabAnonymousCtor___spec__4___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_elabSubst___lambda__6___closed__8; LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabLeadingParserMacro___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_ResolveName_resolveNamespace(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_expandTuple_declRange__1___closed__5; @@ -503,6 +504,7 @@ static lean_object* l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__10; static lean_object* l___regBuiltin_Lean_Elab_Term_elabTrailingParserMacro_declRange__1___closed__3; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_expandCDot_x3f___spec__6(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_expandCDot_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_elabSubst___lambda__6___closed__7; static lean_object* l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__2; static lean_object* l_Lean_Elab_Term_elabCDotFunctionAlias_x3f___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Term_elabShow__1___closed__1; @@ -652,6 +654,7 @@ static lean_object* l___regBuiltin_Lean_Elab_Term_expandShow_declRange__1___clos static lean_object* l___regBuiltin_Lean_Elab_Term_elabHaveI_declRange__1___closed__1; static lean_object* l_Lean_Elab_Term_expandDbgTrace___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Term_elabRunElab_declRange__1___closed__5; +static lean_object* l_Lean_Elab_Term_elabSubst___lambda__6___closed__9; static lean_object* l_Lean_getConstInfoCtor___at_Lean_Elab_Term_elabAnonymousCtor___spec__1___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Term_expandUnreachable_declRange__1___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Term_elabSorry__1___closed__1; @@ -816,7 +819,6 @@ static lean_object* l_Lean_Elab_Term_expandAssert___closed__10; static lean_object* l_Lean_Elab_Term_elabStateRefT___lambda__1___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_BuiltinNotation_0__Lean_Elab_Term_elabParserMacroAux(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_setImplementedBy___at_Lean_Elab_Term_elabUnsafe___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_expandSuffices___closed__9; static lean_object* l___regBuiltin_Lean_Elab_Term_expandDbgTrace_declRange__1___closed__2; LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_BuiltinNotation_0__Lean_Elab_Term_isSubstCandidate___spec__16(lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabSubst___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -918,7 +920,6 @@ static lean_object* l_Lean_Elab_Term_elabAnonymousCtor___closed__2; LEAN_EXPORT lean_object* l_Array_isEqvAux___at_Lean_Elab_Term_elabCDotFunctionAlias_x3f___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__6; static lean_object* l___regBuiltin_Lean_Elab_Term_elabCoeFunNotation_declRange__1___closed__5; -static lean_object* l_Lean_Elab_Term_expandSuffices___closed__8; lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_expandAssert___closed__1; LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Elab_BuiltinNotation_0__Lean_Elab_Term_isSubstCandidate___spec__2___boxed(lean_object*, lean_object*, lean_object*); @@ -1091,6 +1092,7 @@ static lean_object* l_Lean_Elab_Term_elabStateRefT___lambda__1___closed__5; static lean_object* l_Lean_Elab_Term_expandHave___lambda__1___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_expandSuffices__1(lean_object*); extern lean_object* l_Lean_Compiler_implementedByAttr; +lean_object* l_Lean_Syntax_setKind(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_expandAssert___closed__6; static lean_object* l_Lean_Elab_Term_elabSubst___lambda__6___closed__3; lean_object* lean_string_append(lean_object*, lean_object*); @@ -1153,7 +1155,6 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_expandShow__1(lean_object static lean_object* l___regBuiltin_Lean_Elab_Term_elabUnsafe_declRange__1___closed__6; static lean_object* l_Lean_Elab_Term_expandUnreachable___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_expandParen(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_expandSuffices___closed__7; static lean_object* l_Lean_Elab_Term_elabPanic___closed__6; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_elabSubst__1(lean_object*); static lean_object* l_Lean_Elab_Term_elabLeadingParserMacro___lambda__1___closed__4; @@ -7878,34 +7879,6 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_expandSuffices___closed__7() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Tactic", 6, 6); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Term_expandSuffices___closed__8() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("tacticSeq", 9, 9); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Term_expandSuffices___closed__9() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l___regBuiltin_Lean_Elab_Term_elabCoe__1___closed__3; -x_2 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__8; -x_3 = l_Lean_Elab_Term_expandSuffices___closed__7; -x_4 = l_Lean_Elab_Term_expandSuffices___closed__8; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; -} -} LEAN_EXPORT lean_object* l_Lean_Elab_Term_expandSuffices(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { @@ -8003,577 +7976,481 @@ return x_31; } else { -lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; -x_32 = l_Lean_Syntax_getArg(x_25, x_8); -x_33 = l_Lean_Syntax_getArg(x_25, x_10); -lean_dec(x_25); -x_34 = l_Lean_Elab_Term_expandSuffices___closed__9; -lean_inc(x_33); -x_35 = l_Lean_Syntax_isOfKind(x_33, x_34); -if (x_35 == 0) -{ -lean_object* x_36; lean_object* x_37; -lean_dec(x_33); -lean_dec(x_32); -lean_dec(x_23); -lean_dec(x_16); -lean_dec(x_9); -lean_dec(x_1); -x_36 = lean_box(1); -x_37 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_37, 0, x_36); -lean_ctor_set(x_37, 1, x_3); -return x_37; -} -else -{ -lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; lean_object* x_42; uint8_t x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; -x_38 = lean_unsigned_to_nat(3u); -x_39 = l_Lean_Syntax_getArg(x_1, x_38); +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; lean_object* x_38; uint8_t x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; +x_32 = lean_unsigned_to_nat(3u); +x_33 = l_Lean_Syntax_getArg(x_1, x_32); lean_dec(x_1); -x_40 = lean_ctor_get(x_2, 5); -x_41 = 0; -x_42 = l_Lean_SourceInfo_fromRef(x_40, x_41); -x_43 = 1; -x_44 = l_Lean_SourceInfo_fromRef(x_9, x_43); +x_34 = l_Lean_Elab_Term_expandShow___closed__9; +x_35 = l_Lean_Syntax_setKind(x_25, x_34); +x_36 = lean_ctor_get(x_2, 5); +x_37 = 0; +x_38 = l_Lean_SourceInfo_fromRef(x_36, x_37); +x_39 = 1; +x_40 = l_Lean_SourceInfo_fromRef(x_9, x_39); lean_dec(x_9); -x_45 = l_Lean_Elab_Term_expandHave___lambda__4___closed__1; -x_46 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_46, 0, x_44); -lean_ctor_set(x_46, 1, x_45); -x_47 = l_Lean_Elab_Term_expandHave___closed__11; -lean_inc(x_42); -x_48 = l_Lean_Syntax_node1(x_42, x_47, x_16); -x_49 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__3; -x_50 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__4; -lean_inc(x_42); -x_51 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_51, 0, x_42); -lean_ctor_set(x_51, 1, x_49); -lean_ctor_set(x_51, 2, x_50); -x_52 = l_Lean_Elab_Term_elabShow___closed__11; -lean_inc(x_42); -x_53 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_53, 0, x_42); -lean_ctor_set(x_53, 1, x_52); -x_54 = l_Lean_Elab_Term_elabShow___closed__10; -lean_inc(x_42); -x_55 = l_Lean_Syntax_node2(x_42, x_54, x_53, x_23); -lean_inc(x_42); -x_56 = l_Lean_Syntax_node1(x_42, x_49, x_55); -x_57 = l_Lean_Elab_Term_elabShow___closed__12; -lean_inc(x_42); -x_58 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_58, 0, x_42); -lean_ctor_set(x_58, 1, x_57); -x_59 = l_Lean_Elab_Term_expandHave___closed__5; -lean_inc(x_42); -x_60 = l_Lean_Syntax_node5(x_42, x_59, x_48, x_51, x_56, x_58, x_39); -x_61 = l_Lean_Elab_Term_expandHave___closed__3; -lean_inc(x_42); -x_62 = l_Lean_Syntax_node1(x_42, x_61, x_60); -x_63 = l_Lean_Elab_Term_elabShow___closed__13; -lean_inc(x_42); -x_64 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_64, 0, x_42); -lean_ctor_set(x_64, 1, x_63); -x_65 = l_Lean_SourceInfo_fromRef(x_32, x_43); -lean_dec(x_32); -x_66 = l_Lean_Elab_Term_expandShow___closed__10; -x_67 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_67, 0, x_65); -lean_ctor_set(x_67, 1, x_66); -x_68 = l_Lean_Elab_Term_expandShow___closed__9; -lean_inc(x_42); -x_69 = l_Lean_Syntax_node2(x_42, x_68, x_67, x_33); -x_70 = l_Lean_Elab_Term_expandHave___closed__1; -x_71 = l_Lean_Syntax_node4(x_42, x_70, x_46, x_62, x_64, x_69); -x_72 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_72, 0, x_71); -lean_ctor_set(x_72, 1, x_3); -return x_72; -} +x_41 = l_Lean_Elab_Term_expandHave___lambda__4___closed__1; +x_42 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_42, 0, x_40); +lean_ctor_set(x_42, 1, x_41); +x_43 = l_Lean_Elab_Term_expandHave___closed__11; +lean_inc(x_38); +x_44 = l_Lean_Syntax_node1(x_38, x_43, x_16); +x_45 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__3; +x_46 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__4; +lean_inc(x_38); +x_47 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_47, 0, x_38); +lean_ctor_set(x_47, 1, x_45); +lean_ctor_set(x_47, 2, x_46); +x_48 = l_Lean_Elab_Term_elabShow___closed__11; +lean_inc(x_38); +x_49 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_49, 0, x_38); +lean_ctor_set(x_49, 1, x_48); +x_50 = l_Lean_Elab_Term_elabShow___closed__10; +lean_inc(x_38); +x_51 = l_Lean_Syntax_node2(x_38, x_50, x_49, x_23); +lean_inc(x_38); +x_52 = l_Lean_Syntax_node1(x_38, x_45, x_51); +x_53 = l_Lean_Elab_Term_elabShow___closed__12; +lean_inc(x_38); +x_54 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_54, 0, x_38); +lean_ctor_set(x_54, 1, x_53); +x_55 = l_Lean_Elab_Term_expandHave___closed__5; +lean_inc(x_38); +x_56 = l_Lean_Syntax_node5(x_38, x_55, x_44, x_47, x_52, x_54, x_33); +x_57 = l_Lean_Elab_Term_expandHave___closed__3; +lean_inc(x_38); +x_58 = l_Lean_Syntax_node1(x_38, x_57, x_56); +x_59 = l_Lean_Elab_Term_elabShow___closed__13; +lean_inc(x_38); +x_60 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_60, 0, x_38); +lean_ctor_set(x_60, 1, x_59); +x_61 = l_Lean_Elab_Term_expandHave___closed__1; +x_62 = l_Lean_Syntax_node4(x_38, x_61, x_42, x_58, x_60, x_35); +x_63 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_63, 0, x_62); +lean_ctor_set(x_63, 1, x_3); +return x_63; } } else { -lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; uint8_t x_77; lean_object* x_78; uint8_t x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; -x_73 = l_Lean_Syntax_getArg(x_25, x_10); +lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; uint8_t x_68; lean_object* x_69; uint8_t x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; +x_64 = l_Lean_Syntax_getArg(x_25, x_10); lean_dec(x_25); -x_74 = lean_unsigned_to_nat(3u); -x_75 = l_Lean_Syntax_getArg(x_1, x_74); -lean_dec(x_1); -x_76 = lean_ctor_get(x_2, 5); -x_77 = 0; -x_78 = l_Lean_SourceInfo_fromRef(x_76, x_77); -x_79 = 1; -x_80 = l_Lean_SourceInfo_fromRef(x_9, x_79); +x_65 = lean_unsigned_to_nat(3u); +x_66 = l_Lean_Syntax_getArg(x_1, x_65); +lean_dec(x_1); +x_67 = lean_ctor_get(x_2, 5); +x_68 = 0; +x_69 = l_Lean_SourceInfo_fromRef(x_67, x_68); +x_70 = 1; +x_71 = l_Lean_SourceInfo_fromRef(x_9, x_70); lean_dec(x_9); -x_81 = l_Lean_Elab_Term_expandHave___lambda__4___closed__1; -x_82 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_82, 0, x_80); -lean_ctor_set(x_82, 1, x_81); -x_83 = l_Lean_Elab_Term_expandHave___closed__11; -lean_inc(x_78); -x_84 = l_Lean_Syntax_node1(x_78, x_83, x_16); -x_85 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__3; -x_86 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__4; -lean_inc(x_78); -x_87 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_87, 0, x_78); -lean_ctor_set(x_87, 1, x_85); -lean_ctor_set(x_87, 2, x_86); -x_88 = l_Lean_Elab_Term_elabShow___closed__11; -lean_inc(x_78); -x_89 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_89, 0, x_78); -lean_ctor_set(x_89, 1, x_88); -x_90 = l_Lean_Elab_Term_elabShow___closed__10; -lean_inc(x_78); -x_91 = l_Lean_Syntax_node2(x_78, x_90, x_89, x_23); -lean_inc(x_78); -x_92 = l_Lean_Syntax_node1(x_78, x_85, x_91); -x_93 = l_Lean_Elab_Term_elabShow___closed__12; -lean_inc(x_78); -x_94 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_94, 0, x_78); -lean_ctor_set(x_94, 1, x_93); -x_95 = l_Lean_Elab_Term_expandHave___closed__5; -lean_inc(x_78); -x_96 = l_Lean_Syntax_node5(x_78, x_95, x_84, x_87, x_92, x_94, x_75); -x_97 = l_Lean_Elab_Term_expandHave___closed__3; -lean_inc(x_78); -x_98 = l_Lean_Syntax_node1(x_78, x_97, x_96); -x_99 = l_Lean_Elab_Term_elabShow___closed__13; -lean_inc(x_78); -x_100 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_100, 0, x_78); -lean_ctor_set(x_100, 1, x_99); -x_101 = l_Lean_Elab_Term_expandHave___closed__1; -x_102 = l_Lean_Syntax_node4(x_78, x_101, x_82, x_98, x_100, x_73); -x_103 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_103, 0, x_102); -lean_ctor_set(x_103, 1, x_3); -return x_103; +x_72 = l_Lean_Elab_Term_expandHave___lambda__4___closed__1; +x_73 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_73, 0, x_71); +lean_ctor_set(x_73, 1, x_72); +x_74 = l_Lean_Elab_Term_expandHave___closed__11; +lean_inc(x_69); +x_75 = l_Lean_Syntax_node1(x_69, x_74, x_16); +x_76 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__3; +x_77 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__4; +lean_inc(x_69); +x_78 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_78, 0, x_69); +lean_ctor_set(x_78, 1, x_76); +lean_ctor_set(x_78, 2, x_77); +x_79 = l_Lean_Elab_Term_elabShow___closed__11; +lean_inc(x_69); +x_80 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_80, 0, x_69); +lean_ctor_set(x_80, 1, x_79); +x_81 = l_Lean_Elab_Term_elabShow___closed__10; +lean_inc(x_69); +x_82 = l_Lean_Syntax_node2(x_69, x_81, x_80, x_23); +lean_inc(x_69); +x_83 = l_Lean_Syntax_node1(x_69, x_76, x_82); +x_84 = l_Lean_Elab_Term_elabShow___closed__12; +lean_inc(x_69); +x_85 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_85, 0, x_69); +lean_ctor_set(x_85, 1, x_84); +x_86 = l_Lean_Elab_Term_expandHave___closed__5; +lean_inc(x_69); +x_87 = l_Lean_Syntax_node5(x_69, x_86, x_75, x_78, x_83, x_85, x_66); +x_88 = l_Lean_Elab_Term_expandHave___closed__3; +lean_inc(x_69); +x_89 = l_Lean_Syntax_node1(x_69, x_88, x_87); +x_90 = l_Lean_Elab_Term_elabShow___closed__13; +lean_inc(x_69); +x_91 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_91, 0, x_69); +lean_ctor_set(x_91, 1, x_90); +x_92 = l_Lean_Elab_Term_expandHave___closed__1; +x_93 = l_Lean_Syntax_node4(x_69, x_92, x_73, x_89, x_91, x_64); +x_94 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_94, 0, x_93); +lean_ctor_set(x_94, 1, x_3); +return x_94; } } } else { -lean_object* x_104; lean_object* x_105; uint8_t x_106; -x_104 = l_Lean_Syntax_getArg(x_16, x_8); +lean_object* x_95; lean_object* x_96; uint8_t x_97; +x_95 = l_Lean_Syntax_getArg(x_16, x_8); lean_dec(x_16); -x_105 = l_Lean_Elab_Term_expandHave___closed__15; -lean_inc(x_104); -x_106 = l_Lean_Syntax_isOfKind(x_104, x_105); -if (x_106 == 0) +x_96 = l_Lean_Elab_Term_expandHave___closed__15; +lean_inc(x_95); +x_97 = l_Lean_Syntax_isOfKind(x_95, x_96); +if (x_97 == 0) { -lean_object* x_107; uint8_t x_108; -x_107 = l_Lean_Elab_Term_expandHave___closed__17; -lean_inc(x_104); -x_108 = l_Lean_Syntax_isOfKind(x_104, x_107); -if (x_108 == 0) +lean_object* x_98; uint8_t x_99; +x_98 = l_Lean_Elab_Term_expandHave___closed__17; +lean_inc(x_95); +x_99 = l_Lean_Syntax_isOfKind(x_95, x_98); +if (x_99 == 0) { -lean_object* x_109; lean_object* x_110; -lean_dec(x_104); +lean_object* x_100; lean_object* x_101; +lean_dec(x_95); lean_dec(x_11); lean_dec(x_9); lean_dec(x_1); -x_109 = lean_box(1); -x_110 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_110, 0, x_109); -lean_ctor_set(x_110, 1, x_3); -return x_110; +x_100 = lean_box(1); +x_101 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_101, 0, x_100); +lean_ctor_set(x_101, 1, x_3); +return x_101; } else { -lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; uint8_t x_116; -x_111 = l_Lean_Syntax_getArg(x_104, x_8); -lean_dec(x_104); -x_112 = l_Lean_Syntax_getArg(x_11, x_10); -x_113 = lean_unsigned_to_nat(2u); -x_114 = l_Lean_Syntax_getArg(x_11, x_113); +lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; uint8_t x_107; +x_102 = l_Lean_Syntax_getArg(x_95, x_8); +lean_dec(x_95); +x_103 = l_Lean_Syntax_getArg(x_11, x_10); +x_104 = lean_unsigned_to_nat(2u); +x_105 = l_Lean_Syntax_getArg(x_11, x_104); lean_dec(x_11); -x_115 = l_Lean_Elab_Term_expandShow___closed__6; -lean_inc(x_114); -x_116 = l_Lean_Syntax_isOfKind(x_114, x_115); -if (x_116 == 0) +x_106 = l_Lean_Elab_Term_expandShow___closed__6; +lean_inc(x_105); +x_107 = l_Lean_Syntax_isOfKind(x_105, x_106); +if (x_107 == 0) { -lean_object* x_117; uint8_t x_118; -x_117 = l_Lean_Elab_Term_expandShow___closed__4; -lean_inc(x_114); -x_118 = l_Lean_Syntax_isOfKind(x_114, x_117); -if (x_118 == 0) +lean_object* x_108; uint8_t x_109; +x_108 = l_Lean_Elab_Term_expandShow___closed__4; +lean_inc(x_105); +x_109 = l_Lean_Syntax_isOfKind(x_105, x_108); +if (x_109 == 0) { -lean_object* x_119; lean_object* x_120; -lean_dec(x_114); -lean_dec(x_112); -lean_dec(x_111); +lean_object* x_110; lean_object* x_111; +lean_dec(x_105); +lean_dec(x_103); +lean_dec(x_102); lean_dec(x_9); lean_dec(x_1); -x_119 = lean_box(1); -x_120 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_120, 0, x_119); -lean_ctor_set(x_120, 1, x_3); -return x_120; +x_110 = lean_box(1); +x_111 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_111, 0, x_110); +lean_ctor_set(x_111, 1, x_3); +return x_111; } else { -lean_object* x_121; lean_object* x_122; lean_object* x_123; uint8_t x_124; -x_121 = l_Lean_Syntax_getArg(x_114, x_8); -x_122 = l_Lean_Syntax_getArg(x_114, x_10); -lean_dec(x_114); -x_123 = l_Lean_Elab_Term_expandSuffices___closed__9; -lean_inc(x_122); -x_124 = l_Lean_Syntax_isOfKind(x_122, x_123); -if (x_124 == 0) -{ -lean_object* x_125; lean_object* x_126; -lean_dec(x_122); -lean_dec(x_121); -lean_dec(x_112); -lean_dec(x_111); -lean_dec(x_9); +lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; uint8_t x_117; lean_object* x_118; uint8_t x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; +x_112 = lean_unsigned_to_nat(3u); +x_113 = l_Lean_Syntax_getArg(x_1, x_112); lean_dec(x_1); -x_125 = lean_box(1); -x_126 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_126, 0, x_125); -lean_ctor_set(x_126, 1, x_3); -return x_126; +x_114 = l_Lean_Elab_Term_expandShow___closed__9; +x_115 = l_Lean_Syntax_setKind(x_105, x_114); +x_116 = lean_ctor_get(x_2, 5); +x_117 = 0; +x_118 = l_Lean_SourceInfo_fromRef(x_116, x_117); +x_119 = 1; +x_120 = l_Lean_SourceInfo_fromRef(x_9, x_119); +lean_dec(x_9); +x_121 = l_Lean_Elab_Term_expandHave___lambda__4___closed__1; +x_122 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_122, 0, x_120); +lean_ctor_set(x_122, 1, x_121); +x_123 = l_Lean_SourceInfo_fromRef(x_102, x_119); +lean_dec(x_102); +x_124 = l_Lean_Elab_Term_expandHave___lambda__2___closed__3; +x_125 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_125, 0, x_123); +lean_ctor_set(x_125, 1, x_124); +lean_inc(x_118); +x_126 = l_Lean_Syntax_node1(x_118, x_98, x_125); +x_127 = l_Lean_Elab_Term_expandHave___closed__11; +lean_inc(x_118); +x_128 = l_Lean_Syntax_node1(x_118, x_127, x_126); +x_129 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__3; +x_130 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__4; +lean_inc(x_118); +x_131 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_131, 0, x_118); +lean_ctor_set(x_131, 1, x_129); +lean_ctor_set(x_131, 2, x_130); +x_132 = l_Lean_Elab_Term_elabShow___closed__11; +lean_inc(x_118); +x_133 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_133, 0, x_118); +lean_ctor_set(x_133, 1, x_132); +x_134 = l_Lean_Elab_Term_elabShow___closed__10; +lean_inc(x_118); +x_135 = l_Lean_Syntax_node2(x_118, x_134, x_133, x_103); +lean_inc(x_118); +x_136 = l_Lean_Syntax_node1(x_118, x_129, x_135); +x_137 = l_Lean_Elab_Term_elabShow___closed__12; +lean_inc(x_118); +x_138 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_138, 0, x_118); +lean_ctor_set(x_138, 1, x_137); +x_139 = l_Lean_Elab_Term_expandHave___closed__5; +lean_inc(x_118); +x_140 = l_Lean_Syntax_node5(x_118, x_139, x_128, x_131, x_136, x_138, x_113); +x_141 = l_Lean_Elab_Term_expandHave___closed__3; +lean_inc(x_118); +x_142 = l_Lean_Syntax_node1(x_118, x_141, x_140); +x_143 = l_Lean_Elab_Term_elabShow___closed__13; +lean_inc(x_118); +x_144 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_144, 0, x_118); +lean_ctor_set(x_144, 1, x_143); +x_145 = l_Lean_Elab_Term_expandHave___closed__1; +x_146 = l_Lean_Syntax_node4(x_118, x_145, x_122, x_142, x_144, x_115); +x_147 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_147, 0, x_146); +lean_ctor_set(x_147, 1, x_3); +return x_147; +} } else { -lean_object* x_127; lean_object* x_128; lean_object* x_129; uint8_t x_130; lean_object* x_131; uint8_t x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; -x_127 = lean_unsigned_to_nat(3u); -x_128 = l_Lean_Syntax_getArg(x_1, x_127); -lean_dec(x_1); -x_129 = lean_ctor_get(x_2, 5); -x_130 = 0; -x_131 = l_Lean_SourceInfo_fromRef(x_129, x_130); -x_132 = 1; -x_133 = l_Lean_SourceInfo_fromRef(x_9, x_132); +lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; uint8_t x_152; lean_object* x_153; uint8_t x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; +x_148 = l_Lean_Syntax_getArg(x_105, x_10); +lean_dec(x_105); +x_149 = lean_unsigned_to_nat(3u); +x_150 = l_Lean_Syntax_getArg(x_1, x_149); +lean_dec(x_1); +x_151 = lean_ctor_get(x_2, 5); +x_152 = 0; +x_153 = l_Lean_SourceInfo_fromRef(x_151, x_152); +x_154 = 1; +x_155 = l_Lean_SourceInfo_fromRef(x_9, x_154); lean_dec(x_9); -x_134 = l_Lean_Elab_Term_expandHave___lambda__4___closed__1; -x_135 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_135, 0, x_133); -lean_ctor_set(x_135, 1, x_134); -x_136 = l_Lean_SourceInfo_fromRef(x_111, x_132); -lean_dec(x_111); -x_137 = l_Lean_Elab_Term_expandHave___lambda__2___closed__3; -x_138 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_138, 0, x_136); -lean_ctor_set(x_138, 1, x_137); -lean_inc(x_131); -x_139 = l_Lean_Syntax_node1(x_131, x_107, x_138); -x_140 = l_Lean_Elab_Term_expandHave___closed__11; -lean_inc(x_131); -x_141 = l_Lean_Syntax_node1(x_131, x_140, x_139); -x_142 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__3; -x_143 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__4; -lean_inc(x_131); -x_144 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_144, 0, x_131); -lean_ctor_set(x_144, 1, x_142); -lean_ctor_set(x_144, 2, x_143); -x_145 = l_Lean_Elab_Term_elabShow___closed__11; -lean_inc(x_131); -x_146 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_146, 0, x_131); -lean_ctor_set(x_146, 1, x_145); -x_147 = l_Lean_Elab_Term_elabShow___closed__10; -lean_inc(x_131); -x_148 = l_Lean_Syntax_node2(x_131, x_147, x_146, x_112); -lean_inc(x_131); -x_149 = l_Lean_Syntax_node1(x_131, x_142, x_148); -x_150 = l_Lean_Elab_Term_elabShow___closed__12; -lean_inc(x_131); -x_151 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_151, 0, x_131); -lean_ctor_set(x_151, 1, x_150); -x_152 = l_Lean_Elab_Term_expandHave___closed__5; -lean_inc(x_131); -x_153 = l_Lean_Syntax_node5(x_131, x_152, x_141, x_144, x_149, x_151, x_128); -x_154 = l_Lean_Elab_Term_expandHave___closed__3; -lean_inc(x_131); -x_155 = l_Lean_Syntax_node1(x_131, x_154, x_153); -x_156 = l_Lean_Elab_Term_elabShow___closed__13; -lean_inc(x_131); +x_156 = l_Lean_Elab_Term_expandHave___lambda__4___closed__1; x_157 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_157, 0, x_131); +lean_ctor_set(x_157, 0, x_155); lean_ctor_set(x_157, 1, x_156); -x_158 = l_Lean_SourceInfo_fromRef(x_121, x_132); -lean_dec(x_121); -x_159 = l_Lean_Elab_Term_expandShow___closed__10; +x_158 = l_Lean_SourceInfo_fromRef(x_102, x_154); +lean_dec(x_102); +x_159 = l_Lean_Elab_Term_expandHave___lambda__2___closed__3; x_160 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_160, 0, x_158); lean_ctor_set(x_160, 1, x_159); -x_161 = l_Lean_Elab_Term_expandShow___closed__9; -lean_inc(x_131); -x_162 = l_Lean_Syntax_node2(x_131, x_161, x_160, x_122); -x_163 = l_Lean_Elab_Term_expandHave___closed__1; -x_164 = l_Lean_Syntax_node4(x_131, x_163, x_135, x_155, x_157, x_162); -x_165 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_165, 0, x_164); -lean_ctor_set(x_165, 1, x_3); -return x_165; -} -} -} -else -{ -lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; uint8_t x_170; lean_object* x_171; uint8_t x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; -x_166 = l_Lean_Syntax_getArg(x_114, x_10); -lean_dec(x_114); -x_167 = lean_unsigned_to_nat(3u); -x_168 = l_Lean_Syntax_getArg(x_1, x_167); -lean_dec(x_1); -x_169 = lean_ctor_get(x_2, 5); -x_170 = 0; -x_171 = l_Lean_SourceInfo_fromRef(x_169, x_170); -x_172 = 1; -x_173 = l_Lean_SourceInfo_fromRef(x_9, x_172); -lean_dec(x_9); -x_174 = l_Lean_Elab_Term_expandHave___lambda__4___closed__1; -x_175 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_175, 0, x_173); -lean_ctor_set(x_175, 1, x_174); -x_176 = l_Lean_SourceInfo_fromRef(x_111, x_172); -lean_dec(x_111); -x_177 = l_Lean_Elab_Term_expandHave___lambda__2___closed__3; -x_178 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_178, 0, x_176); -lean_ctor_set(x_178, 1, x_177); -lean_inc(x_171); -x_179 = l_Lean_Syntax_node1(x_171, x_107, x_178); -x_180 = l_Lean_Elab_Term_expandHave___closed__11; -lean_inc(x_171); -x_181 = l_Lean_Syntax_node1(x_171, x_180, x_179); -x_182 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__3; -x_183 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__4; -lean_inc(x_171); -x_184 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_184, 0, x_171); -lean_ctor_set(x_184, 1, x_182); -lean_ctor_set(x_184, 2, x_183); -x_185 = l_Lean_Elab_Term_elabShow___closed__11; -lean_inc(x_171); -x_186 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_186, 0, x_171); -lean_ctor_set(x_186, 1, x_185); -x_187 = l_Lean_Elab_Term_elabShow___closed__10; -lean_inc(x_171); -x_188 = l_Lean_Syntax_node2(x_171, x_187, x_186, x_112); -lean_inc(x_171); -x_189 = l_Lean_Syntax_node1(x_171, x_182, x_188); -x_190 = l_Lean_Elab_Term_elabShow___closed__12; -lean_inc(x_171); -x_191 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_191, 0, x_171); -lean_ctor_set(x_191, 1, x_190); -x_192 = l_Lean_Elab_Term_expandHave___closed__5; -lean_inc(x_171); -x_193 = l_Lean_Syntax_node5(x_171, x_192, x_181, x_184, x_189, x_191, x_168); -x_194 = l_Lean_Elab_Term_expandHave___closed__3; -lean_inc(x_171); -x_195 = l_Lean_Syntax_node1(x_171, x_194, x_193); -x_196 = l_Lean_Elab_Term_elabShow___closed__13; -lean_inc(x_171); -x_197 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_197, 0, x_171); -lean_ctor_set(x_197, 1, x_196); -x_198 = l_Lean_Elab_Term_expandHave___closed__1; -x_199 = l_Lean_Syntax_node4(x_171, x_198, x_175, x_195, x_197, x_166); -x_200 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_200, 0, x_199); -lean_ctor_set(x_200, 1, x_3); -return x_200; +lean_inc(x_153); +x_161 = l_Lean_Syntax_node1(x_153, x_98, x_160); +x_162 = l_Lean_Elab_Term_expandHave___closed__11; +lean_inc(x_153); +x_163 = l_Lean_Syntax_node1(x_153, x_162, x_161); +x_164 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__3; +x_165 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__4; +lean_inc(x_153); +x_166 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_166, 0, x_153); +lean_ctor_set(x_166, 1, x_164); +lean_ctor_set(x_166, 2, x_165); +x_167 = l_Lean_Elab_Term_elabShow___closed__11; +lean_inc(x_153); +x_168 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_168, 0, x_153); +lean_ctor_set(x_168, 1, x_167); +x_169 = l_Lean_Elab_Term_elabShow___closed__10; +lean_inc(x_153); +x_170 = l_Lean_Syntax_node2(x_153, x_169, x_168, x_103); +lean_inc(x_153); +x_171 = l_Lean_Syntax_node1(x_153, x_164, x_170); +x_172 = l_Lean_Elab_Term_elabShow___closed__12; +lean_inc(x_153); +x_173 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_173, 0, x_153); +lean_ctor_set(x_173, 1, x_172); +x_174 = l_Lean_Elab_Term_expandHave___closed__5; +lean_inc(x_153); +x_175 = l_Lean_Syntax_node5(x_153, x_174, x_163, x_166, x_171, x_173, x_150); +x_176 = l_Lean_Elab_Term_expandHave___closed__3; +lean_inc(x_153); +x_177 = l_Lean_Syntax_node1(x_153, x_176, x_175); +x_178 = l_Lean_Elab_Term_elabShow___closed__13; +lean_inc(x_153); +x_179 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_179, 0, x_153); +lean_ctor_set(x_179, 1, x_178); +x_180 = l_Lean_Elab_Term_expandHave___closed__1; +x_181 = l_Lean_Syntax_node4(x_153, x_180, x_157, x_177, x_179, x_148); +x_182 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_182, 0, x_181); +lean_ctor_set(x_182, 1, x_3); +return x_182; } } } else { -lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; uint8_t x_205; -x_201 = l_Lean_Syntax_getArg(x_11, x_10); -x_202 = lean_unsigned_to_nat(2u); -x_203 = l_Lean_Syntax_getArg(x_11, x_202); +lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; uint8_t x_187; +x_183 = l_Lean_Syntax_getArg(x_11, x_10); +x_184 = lean_unsigned_to_nat(2u); +x_185 = l_Lean_Syntax_getArg(x_11, x_184); lean_dec(x_11); -x_204 = l_Lean_Elab_Term_expandShow___closed__6; -lean_inc(x_203); -x_205 = l_Lean_Syntax_isOfKind(x_203, x_204); -if (x_205 == 0) -{ -lean_object* x_206; uint8_t x_207; -x_206 = l_Lean_Elab_Term_expandShow___closed__4; -lean_inc(x_203); -x_207 = l_Lean_Syntax_isOfKind(x_203, x_206); -if (x_207 == 0) -{ -lean_object* x_208; lean_object* x_209; -lean_dec(x_203); -lean_dec(x_201); -lean_dec(x_104); -lean_dec(x_9); -lean_dec(x_1); -x_208 = lean_box(1); -x_209 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_209, 0, x_208); -lean_ctor_set(x_209, 1, x_3); -return x_209; -} -else -{ -lean_object* x_210; lean_object* x_211; lean_object* x_212; uint8_t x_213; -x_210 = l_Lean_Syntax_getArg(x_203, x_8); -x_211 = l_Lean_Syntax_getArg(x_203, x_10); -lean_dec(x_203); -x_212 = l_Lean_Elab_Term_expandSuffices___closed__9; -lean_inc(x_211); -x_213 = l_Lean_Syntax_isOfKind(x_211, x_212); -if (x_213 == 0) +x_186 = l_Lean_Elab_Term_expandShow___closed__6; +lean_inc(x_185); +x_187 = l_Lean_Syntax_isOfKind(x_185, x_186); +if (x_187 == 0) +{ +lean_object* x_188; uint8_t x_189; +x_188 = l_Lean_Elab_Term_expandShow___closed__4; +lean_inc(x_185); +x_189 = l_Lean_Syntax_isOfKind(x_185, x_188); +if (x_189 == 0) { -lean_object* x_214; lean_object* x_215; -lean_dec(x_211); -lean_dec(x_210); -lean_dec(x_201); -lean_dec(x_104); +lean_object* x_190; lean_object* x_191; +lean_dec(x_185); +lean_dec(x_183); +lean_dec(x_95); lean_dec(x_9); lean_dec(x_1); -x_214 = lean_box(1); -x_215 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_215, 0, x_214); -lean_ctor_set(x_215, 1, x_3); -return x_215; +x_190 = lean_box(1); +x_191 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_191, 0, x_190); +lean_ctor_set(x_191, 1, x_3); +return x_191; } else { -lean_object* x_216; lean_object* x_217; lean_object* x_218; uint8_t x_219; lean_object* x_220; uint8_t x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; -x_216 = lean_unsigned_to_nat(3u); -x_217 = l_Lean_Syntax_getArg(x_1, x_216); +lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; uint8_t x_197; lean_object* x_198; uint8_t x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; +x_192 = lean_unsigned_to_nat(3u); +x_193 = l_Lean_Syntax_getArg(x_1, x_192); lean_dec(x_1); -x_218 = lean_ctor_get(x_2, 5); -x_219 = 0; -x_220 = l_Lean_SourceInfo_fromRef(x_218, x_219); -x_221 = 1; -x_222 = l_Lean_SourceInfo_fromRef(x_9, x_221); +x_194 = l_Lean_Elab_Term_expandShow___closed__9; +x_195 = l_Lean_Syntax_setKind(x_185, x_194); +x_196 = lean_ctor_get(x_2, 5); +x_197 = 0; +x_198 = l_Lean_SourceInfo_fromRef(x_196, x_197); +x_199 = 1; +x_200 = l_Lean_SourceInfo_fromRef(x_9, x_199); lean_dec(x_9); -x_223 = l_Lean_Elab_Term_expandHave___lambda__4___closed__1; -x_224 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_224, 0, x_222); -lean_ctor_set(x_224, 1, x_223); -x_225 = l_Lean_Elab_Term_expandHave___closed__11; -lean_inc(x_220); -x_226 = l_Lean_Syntax_node1(x_220, x_225, x_104); -x_227 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__3; -x_228 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__4; -lean_inc(x_220); -x_229 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_229, 0, x_220); -lean_ctor_set(x_229, 1, x_227); -lean_ctor_set(x_229, 2, x_228); -x_230 = l_Lean_Elab_Term_elabShow___closed__11; -lean_inc(x_220); -x_231 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_231, 0, x_220); -lean_ctor_set(x_231, 1, x_230); -x_232 = l_Lean_Elab_Term_elabShow___closed__10; -lean_inc(x_220); -x_233 = l_Lean_Syntax_node2(x_220, x_232, x_231, x_201); -lean_inc(x_220); -x_234 = l_Lean_Syntax_node1(x_220, x_227, x_233); -x_235 = l_Lean_Elab_Term_elabShow___closed__12; -lean_inc(x_220); -x_236 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_236, 0, x_220); -lean_ctor_set(x_236, 1, x_235); -x_237 = l_Lean_Elab_Term_expandHave___closed__5; -lean_inc(x_220); -x_238 = l_Lean_Syntax_node5(x_220, x_237, x_226, x_229, x_234, x_236, x_217); -x_239 = l_Lean_Elab_Term_expandHave___closed__3; -lean_inc(x_220); -x_240 = l_Lean_Syntax_node1(x_220, x_239, x_238); -x_241 = l_Lean_Elab_Term_elabShow___closed__13; -lean_inc(x_220); -x_242 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_242, 0, x_220); -lean_ctor_set(x_242, 1, x_241); -x_243 = l_Lean_SourceInfo_fromRef(x_210, x_221); -lean_dec(x_210); -x_244 = l_Lean_Elab_Term_expandShow___closed__10; +x_201 = l_Lean_Elab_Term_expandHave___lambda__4___closed__1; +x_202 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_202, 0, x_200); +lean_ctor_set(x_202, 1, x_201); +x_203 = l_Lean_Elab_Term_expandHave___closed__11; +lean_inc(x_198); +x_204 = l_Lean_Syntax_node1(x_198, x_203, x_95); +x_205 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__3; +x_206 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__4; +lean_inc(x_198); +x_207 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_207, 0, x_198); +lean_ctor_set(x_207, 1, x_205); +lean_ctor_set(x_207, 2, x_206); +x_208 = l_Lean_Elab_Term_elabShow___closed__11; +lean_inc(x_198); +x_209 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_209, 0, x_198); +lean_ctor_set(x_209, 1, x_208); +x_210 = l_Lean_Elab_Term_elabShow___closed__10; +lean_inc(x_198); +x_211 = l_Lean_Syntax_node2(x_198, x_210, x_209, x_183); +lean_inc(x_198); +x_212 = l_Lean_Syntax_node1(x_198, x_205, x_211); +x_213 = l_Lean_Elab_Term_elabShow___closed__12; +lean_inc(x_198); +x_214 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_214, 0, x_198); +lean_ctor_set(x_214, 1, x_213); +x_215 = l_Lean_Elab_Term_expandHave___closed__5; +lean_inc(x_198); +x_216 = l_Lean_Syntax_node5(x_198, x_215, x_204, x_207, x_212, x_214, x_193); +x_217 = l_Lean_Elab_Term_expandHave___closed__3; +lean_inc(x_198); +x_218 = l_Lean_Syntax_node1(x_198, x_217, x_216); +x_219 = l_Lean_Elab_Term_elabShow___closed__13; +lean_inc(x_198); +x_220 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_220, 0, x_198); +lean_ctor_set(x_220, 1, x_219); +x_221 = l_Lean_Elab_Term_expandHave___closed__1; +x_222 = l_Lean_Syntax_node4(x_198, x_221, x_202, x_218, x_220, x_195); +x_223 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_223, 0, x_222); +lean_ctor_set(x_223, 1, x_3); +return x_223; +} +} +else +{ +lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; uint8_t x_228; lean_object* x_229; uint8_t x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; +x_224 = l_Lean_Syntax_getArg(x_185, x_10); +lean_dec(x_185); +x_225 = lean_unsigned_to_nat(3u); +x_226 = l_Lean_Syntax_getArg(x_1, x_225); +lean_dec(x_1); +x_227 = lean_ctor_get(x_2, 5); +x_228 = 0; +x_229 = l_Lean_SourceInfo_fromRef(x_227, x_228); +x_230 = 1; +x_231 = l_Lean_SourceInfo_fromRef(x_9, x_230); +lean_dec(x_9); +x_232 = l_Lean_Elab_Term_expandHave___lambda__4___closed__1; +x_233 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_233, 0, x_231); +lean_ctor_set(x_233, 1, x_232); +x_234 = l_Lean_Elab_Term_expandHave___closed__11; +lean_inc(x_229); +x_235 = l_Lean_Syntax_node1(x_229, x_234, x_95); +x_236 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__3; +x_237 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__4; +lean_inc(x_229); +x_238 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_238, 0, x_229); +lean_ctor_set(x_238, 1, x_236); +lean_ctor_set(x_238, 2, x_237); +x_239 = l_Lean_Elab_Term_elabShow___closed__11; +lean_inc(x_229); +x_240 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_240, 0, x_229); +lean_ctor_set(x_240, 1, x_239); +x_241 = l_Lean_Elab_Term_elabShow___closed__10; +lean_inc(x_229); +x_242 = l_Lean_Syntax_node2(x_229, x_241, x_240, x_183); +lean_inc(x_229); +x_243 = l_Lean_Syntax_node1(x_229, x_236, x_242); +x_244 = l_Lean_Elab_Term_elabShow___closed__12; +lean_inc(x_229); x_245 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_245, 0, x_243); +lean_ctor_set(x_245, 0, x_229); lean_ctor_set(x_245, 1, x_244); -x_246 = l_Lean_Elab_Term_expandShow___closed__9; -lean_inc(x_220); -x_247 = l_Lean_Syntax_node2(x_220, x_246, x_245, x_211); -x_248 = l_Lean_Elab_Term_expandHave___closed__1; -x_249 = l_Lean_Syntax_node4(x_220, x_248, x_224, x_240, x_242, x_247); -x_250 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_250, 0, x_249); -lean_ctor_set(x_250, 1, x_3); -return x_250; -} -} -} -else -{ -lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; uint8_t x_255; lean_object* x_256; uint8_t x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; -x_251 = l_Lean_Syntax_getArg(x_203, x_10); -lean_dec(x_203); -x_252 = lean_unsigned_to_nat(3u); -x_253 = l_Lean_Syntax_getArg(x_1, x_252); -lean_dec(x_1); -x_254 = lean_ctor_get(x_2, 5); -x_255 = 0; -x_256 = l_Lean_SourceInfo_fromRef(x_254, x_255); -x_257 = 1; -x_258 = l_Lean_SourceInfo_fromRef(x_9, x_257); -lean_dec(x_9); -x_259 = l_Lean_Elab_Term_expandHave___lambda__4___closed__1; -x_260 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_260, 0, x_258); -lean_ctor_set(x_260, 1, x_259); -x_261 = l_Lean_Elab_Term_expandHave___closed__11; -lean_inc(x_256); -x_262 = l_Lean_Syntax_node1(x_256, x_261, x_104); -x_263 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__3; -x_264 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__4; -lean_inc(x_256); -x_265 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_265, 0, x_256); -lean_ctor_set(x_265, 1, x_263); -lean_ctor_set(x_265, 2, x_264); -x_266 = l_Lean_Elab_Term_elabShow___closed__11; -lean_inc(x_256); -x_267 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_267, 0, x_256); -lean_ctor_set(x_267, 1, x_266); -x_268 = l_Lean_Elab_Term_elabShow___closed__10; -lean_inc(x_256); -x_269 = l_Lean_Syntax_node2(x_256, x_268, x_267, x_201); -lean_inc(x_256); -x_270 = l_Lean_Syntax_node1(x_256, x_263, x_269); -x_271 = l_Lean_Elab_Term_elabShow___closed__12; -lean_inc(x_256); -x_272 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_272, 0, x_256); -lean_ctor_set(x_272, 1, x_271); -x_273 = l_Lean_Elab_Term_expandHave___closed__5; -lean_inc(x_256); -x_274 = l_Lean_Syntax_node5(x_256, x_273, x_262, x_265, x_270, x_272, x_253); -x_275 = l_Lean_Elab_Term_expandHave___closed__3; -lean_inc(x_256); -x_276 = l_Lean_Syntax_node1(x_256, x_275, x_274); -x_277 = l_Lean_Elab_Term_elabShow___closed__13; -lean_inc(x_256); -x_278 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_278, 0, x_256); -lean_ctor_set(x_278, 1, x_277); -x_279 = l_Lean_Elab_Term_expandHave___closed__1; -x_280 = l_Lean_Syntax_node4(x_256, x_279, x_260, x_276, x_278, x_251); -x_281 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_281, 0, x_280); -lean_ctor_set(x_281, 1, x_3); -return x_281; +x_246 = l_Lean_Elab_Term_expandHave___closed__5; +lean_inc(x_229); +x_247 = l_Lean_Syntax_node5(x_229, x_246, x_235, x_238, x_243, x_245, x_226); +x_248 = l_Lean_Elab_Term_expandHave___closed__3; +lean_inc(x_229); +x_249 = l_Lean_Syntax_node1(x_229, x_248, x_247); +x_250 = l_Lean_Elab_Term_elabShow___closed__13; +lean_inc(x_229); +x_251 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_251, 0, x_229); +lean_ctor_set(x_251, 1, x_250); +x_252 = l_Lean_Elab_Term_expandHave___closed__1; +x_253 = l_Lean_Syntax_node4(x_229, x_252, x_233, x_249, x_251, x_224); +x_254 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_254, 0, x_253); +lean_ctor_set(x_254, 1, x_3); +return x_254; } } } @@ -24958,23 +24835,51 @@ static lean_object* _init_l_Lean_Elab_Term_elabSubst___lambda__6___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("tacticSeq1Indented", 18, 18); +x_1 = lean_mk_string_unchecked("Tactic", 6, 6); return x_1; } } static lean_object* _init_l_Lean_Elab_Term_elabSubst___lambda__6___closed__2() { _start: { +lean_object* x_1; +x_1 = lean_mk_string_unchecked("tacticSeq", 9, 9); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Term_elabSubst___lambda__6___closed__3() { +_start: +{ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l___regBuiltin_Lean_Elab_Term_elabCoe__1___closed__3; x_2 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__8; -x_3 = l_Lean_Elab_Term_expandSuffices___closed__7; -x_4 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__1; +x_3 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__1; +x_4 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__2; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Elab_Term_elabSubst___lambda__6___closed__3() { +static lean_object* _init_l_Lean_Elab_Term_elabSubst___lambda__6___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("tacticSeq1Indented", 18, 18); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Term_elabSubst___lambda__6___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l___regBuiltin_Lean_Elab_Term_elabCoe__1___closed__3; +x_2 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__8; +x_3 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__1; +x_4 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__4; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Elab_Term_elabSubst___lambda__6___closed__6() { _start: { lean_object* x_1; @@ -24982,19 +24887,19 @@ x_1 = lean_mk_string_unchecked("subst", 5, 5); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_elabSubst___lambda__6___closed__4() { +static lean_object* _init_l_Lean_Elab_Term_elabSubst___lambda__6___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l___regBuiltin_Lean_Elab_Term_elabCoe__1___closed__3; x_2 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__8; -x_3 = l_Lean_Elab_Term_expandSuffices___closed__7; -x_4 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__3; +x_3 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__1; +x_4 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__6; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Elab_Term_elabSubst___lambda__6___closed__5() { +static lean_object* _init_l_Lean_Elab_Term_elabSubst___lambda__6___closed__8() { _start: { lean_object* x_1; @@ -25002,14 +24907,14 @@ x_1 = lean_mk_string_unchecked("exact", 5, 5); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_elabSubst___lambda__6___closed__6() { +static lean_object* _init_l_Lean_Elab_Term_elabSubst___lambda__6___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l___regBuiltin_Lean_Elab_Term_elabCoe__1___closed__3; x_2 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__8; -x_3 = l_Lean_Elab_Term_expandSuffices___closed__7; -x_4 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__5; +x_3 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__1; +x_4 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__8; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } @@ -25036,7 +24941,7 @@ lean_inc(x_14); lean_ctor_set_tag(x_15, 2); lean_ctor_set(x_15, 1, x_19); lean_ctor_set(x_15, 0, x_14); -x_20 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__3; +x_20 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__6; lean_inc(x_14); x_21 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_21, 0, x_14); @@ -25044,7 +24949,7 @@ lean_ctor_set(x_21, 1, x_20); x_22 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__3; lean_inc(x_14); x_23 = l_Lean_Syntax_node1(x_14, x_22, x_1); -x_24 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__4; +x_24 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__7; lean_inc(x_14); x_25 = l_Lean_Syntax_node2(x_14, x_24, x_21, x_23); x_26 = l_Lean_Elab_Term_elabShow___closed__13; @@ -25052,20 +24957,20 @@ lean_inc(x_14); x_27 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_27, 0, x_14); lean_ctor_set(x_27, 1, x_26); -x_28 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__5; +x_28 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__8; lean_inc(x_14); x_29 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_29, 0, x_14); lean_ctor_set(x_29, 1, x_28); -x_30 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__6; +x_30 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__9; lean_inc(x_14); x_31 = l_Lean_Syntax_node2(x_14, x_30, x_29, x_4); lean_inc(x_14); x_32 = l_Lean_Syntax_node3(x_14, x_22, x_25, x_27, x_31); -x_33 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__2; +x_33 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__5; lean_inc(x_14); x_34 = l_Lean_Syntax_node1(x_14, x_33, x_32); -x_35 = l_Lean_Elab_Term_expandSuffices___closed__9; +x_35 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__3; lean_inc(x_14); x_36 = l_Lean_Syntax_node1(x_14, x_35, x_34); x_37 = l_Lean_Elab_Term_expandShow___closed__9; @@ -25095,7 +25000,7 @@ lean_inc(x_14); x_47 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_47, 0, x_14); lean_ctor_set(x_47, 1, x_46); -x_48 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__3; +x_48 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__6; lean_inc(x_14); x_49 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_49, 0, x_14); @@ -25103,7 +25008,7 @@ lean_ctor_set(x_49, 1, x_48); x_50 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__3; lean_inc(x_14); x_51 = l_Lean_Syntax_node1(x_14, x_50, x_1); -x_52 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__4; +x_52 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__7; lean_inc(x_14); x_53 = l_Lean_Syntax_node2(x_14, x_52, x_49, x_51); x_54 = l_Lean_Elab_Term_elabShow___closed__13; @@ -25111,20 +25016,20 @@ lean_inc(x_14); x_55 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_55, 0, x_14); lean_ctor_set(x_55, 1, x_54); -x_56 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__5; +x_56 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__8; lean_inc(x_14); x_57 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_57, 0, x_14); lean_ctor_set(x_57, 1, x_56); -x_58 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__6; +x_58 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__9; lean_inc(x_14); x_59 = l_Lean_Syntax_node2(x_14, x_58, x_57, x_4); lean_inc(x_14); x_60 = l_Lean_Syntax_node3(x_14, x_50, x_53, x_55, x_59); -x_61 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__2; +x_61 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__5; lean_inc(x_14); x_62 = l_Lean_Syntax_node1(x_14, x_61, x_60); -x_63 = l_Lean_Elab_Term_expandSuffices___closed__9; +x_63 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__3; lean_inc(x_14); x_64 = l_Lean_Syntax_node1(x_14, x_63, x_62); x_65 = l_Lean_Elab_Term_expandShow___closed__9; @@ -25190,7 +25095,7 @@ lean_inc(x_22); lean_ctor_set_tag(x_23, 2); lean_ctor_set(x_23, 1, x_27); lean_ctor_set(x_23, 0, x_22); -x_28 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__3; +x_28 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__6; lean_inc(x_22); lean_ctor_set_tag(x_13, 2); lean_ctor_set(x_13, 1, x_28); @@ -25198,7 +25103,7 @@ lean_ctor_set(x_13, 0, x_22); x_29 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__3; lean_inc(x_22); x_30 = l_Lean_Syntax_node1(x_22, x_29, x_5); -x_31 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__4; +x_31 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__7; lean_inc(x_22); x_32 = l_Lean_Syntax_node2(x_22, x_31, x_13, x_30); x_33 = l_Lean_Elab_Term_elabShow___closed__13; @@ -25206,20 +25111,20 @@ lean_inc(x_22); x_34 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_34, 0, x_22); lean_ctor_set(x_34, 1, x_33); -x_35 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__5; +x_35 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__8; lean_inc(x_22); x_36 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_36, 0, x_22); lean_ctor_set(x_36, 1, x_35); -x_37 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__6; +x_37 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__9; lean_inc(x_22); x_38 = l_Lean_Syntax_node2(x_22, x_37, x_36, x_4); lean_inc(x_22); x_39 = l_Lean_Syntax_node3(x_22, x_29, x_32, x_34, x_38); -x_40 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__2; +x_40 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__5; lean_inc(x_22); x_41 = l_Lean_Syntax_node1(x_22, x_40, x_39); -x_42 = l_Lean_Elab_Term_expandSuffices___closed__9; +x_42 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__3; lean_inc(x_22); x_43 = l_Lean_Syntax_node1(x_22, x_42, x_41); x_44 = l_Lean_Elab_Term_expandShow___closed__9; @@ -25249,7 +25154,7 @@ lean_inc(x_22); x_54 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_54, 0, x_22); lean_ctor_set(x_54, 1, x_53); -x_55 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__3; +x_55 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__6; lean_inc(x_22); lean_ctor_set_tag(x_13, 2); lean_ctor_set(x_13, 1, x_55); @@ -25257,7 +25162,7 @@ lean_ctor_set(x_13, 0, x_22); x_56 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__3; lean_inc(x_22); x_57 = l_Lean_Syntax_node1(x_22, x_56, x_5); -x_58 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__4; +x_58 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__7; lean_inc(x_22); x_59 = l_Lean_Syntax_node2(x_22, x_58, x_13, x_57); x_60 = l_Lean_Elab_Term_elabShow___closed__13; @@ -25265,20 +25170,20 @@ lean_inc(x_22); x_61 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_61, 0, x_22); lean_ctor_set(x_61, 1, x_60); -x_62 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__5; +x_62 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__8; lean_inc(x_22); x_63 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_63, 0, x_22); lean_ctor_set(x_63, 1, x_62); -x_64 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__6; +x_64 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__9; lean_inc(x_22); x_65 = l_Lean_Syntax_node2(x_22, x_64, x_63, x_4); lean_inc(x_22); x_66 = l_Lean_Syntax_node3(x_22, x_56, x_59, x_61, x_65); -x_67 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__2; +x_67 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__5; lean_inc(x_22); x_68 = l_Lean_Syntax_node1(x_22, x_67, x_66); -x_69 = l_Lean_Elab_Term_expandSuffices___closed__9; +x_69 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__3; lean_inc(x_22); x_70 = l_Lean_Syntax_node1(x_22, x_69, x_68); x_71 = l_Lean_Elab_Term_expandShow___closed__9; @@ -25348,7 +25253,7 @@ if (lean_is_scalar(x_89)) { } lean_ctor_set(x_91, 0, x_86); lean_ctor_set(x_91, 1, x_90); -x_92 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__3; +x_92 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__6; lean_inc(x_86); x_93 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_93, 0, x_86); @@ -25356,7 +25261,7 @@ lean_ctor_set(x_93, 1, x_92); x_94 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__3; lean_inc(x_86); x_95 = l_Lean_Syntax_node1(x_86, x_94, x_5); -x_96 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__4; +x_96 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__7; lean_inc(x_86); x_97 = l_Lean_Syntax_node2(x_86, x_96, x_93, x_95); x_98 = l_Lean_Elab_Term_elabShow___closed__13; @@ -25364,20 +25269,20 @@ lean_inc(x_86); x_99 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_99, 0, x_86); lean_ctor_set(x_99, 1, x_98); -x_100 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__5; +x_100 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__8; lean_inc(x_86); x_101 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_101, 0, x_86); lean_ctor_set(x_101, 1, x_100); -x_102 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__6; +x_102 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__9; lean_inc(x_86); x_103 = l_Lean_Syntax_node2(x_86, x_102, x_101, x_4); lean_inc(x_86); x_104 = l_Lean_Syntax_node3(x_86, x_94, x_97, x_99, x_103); -x_105 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__2; +x_105 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__5; lean_inc(x_86); x_106 = l_Lean_Syntax_node1(x_86, x_105, x_104); -x_107 = l_Lean_Elab_Term_expandSuffices___closed__9; +x_107 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__3; lean_inc(x_86); x_108 = l_Lean_Syntax_node1(x_86, x_107, x_106); x_109 = l_Lean_Elab_Term_expandShow___closed__9; @@ -27064,7 +26969,7 @@ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_obj x_1 = l___regBuiltin_Lean_Elab_Term_elabCoe__1___closed__3; x_2 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__8; x_3 = l___regBuiltin_Lean_Elab_Term_elabCoe__1___closed__5; -x_4 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__3; +x_4 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__6; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } @@ -31442,7 +31347,7 @@ static lean_object* _init_l_Lean_Elab_Term_elabUnsafe___lambda__1___closed__6() lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Elab_Term_elabUnsafe___lambda__1___closed__3; x_2 = l_Lean_Elab_Term_elabUnsafe___lambda__1___closed__4; -x_3 = lean_unsigned_to_nat(493u); +x_3 = lean_unsigned_to_nat(501u); x_4 = lean_unsigned_to_nat(54u); x_5 = l_Lean_Elab_Term_elabUnsafe___lambda__1___closed__5; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -31455,7 +31360,7 @@ static lean_object* _init_l_Lean_Elab_Term_elabUnsafe___lambda__1___closed__7() lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Elab_Term_elabUnsafe___lambda__1___closed__3; x_2 = l_Lean_Elab_Term_elabUnsafe___lambda__1___closed__4; -x_3 = lean_unsigned_to_nat(494u); +x_3 = lean_unsigned_to_nat(502u); x_4 = lean_unsigned_to_nat(55u); x_5 = l_Lean_Elab_Term_elabUnsafe___lambda__1___closed__5; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -35202,12 +35107,6 @@ l_Lean_Elab_Term_expandSuffices___closed__5 = _init_l_Lean_Elab_Term_expandSuffi lean_mark_persistent(l_Lean_Elab_Term_expandSuffices___closed__5); l_Lean_Elab_Term_expandSuffices___closed__6 = _init_l_Lean_Elab_Term_expandSuffices___closed__6(); lean_mark_persistent(l_Lean_Elab_Term_expandSuffices___closed__6); -l_Lean_Elab_Term_expandSuffices___closed__7 = _init_l_Lean_Elab_Term_expandSuffices___closed__7(); -lean_mark_persistent(l_Lean_Elab_Term_expandSuffices___closed__7); -l_Lean_Elab_Term_expandSuffices___closed__8 = _init_l_Lean_Elab_Term_expandSuffices___closed__8(); -lean_mark_persistent(l_Lean_Elab_Term_expandSuffices___closed__8); -l_Lean_Elab_Term_expandSuffices___closed__9 = _init_l_Lean_Elab_Term_expandSuffices___closed__9(); -lean_mark_persistent(l_Lean_Elab_Term_expandSuffices___closed__9); l___regBuiltin_Lean_Elab_Term_expandSuffices__1___closed__1 = _init_l___regBuiltin_Lean_Elab_Term_expandSuffices__1___closed__1(); lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_expandSuffices__1___closed__1); l___regBuiltin_Lean_Elab_Term_expandSuffices__1___closed__2 = _init_l___regBuiltin_Lean_Elab_Term_expandSuffices__1___closed__2(); @@ -35970,6 +35869,12 @@ l_Lean_Elab_Term_elabSubst___lambda__6___closed__5 = _init_l_Lean_Elab_Term_elab lean_mark_persistent(l_Lean_Elab_Term_elabSubst___lambda__6___closed__5); l_Lean_Elab_Term_elabSubst___lambda__6___closed__6 = _init_l_Lean_Elab_Term_elabSubst___lambda__6___closed__6(); lean_mark_persistent(l_Lean_Elab_Term_elabSubst___lambda__6___closed__6); +l_Lean_Elab_Term_elabSubst___lambda__6___closed__7 = _init_l_Lean_Elab_Term_elabSubst___lambda__6___closed__7(); +lean_mark_persistent(l_Lean_Elab_Term_elabSubst___lambda__6___closed__7); +l_Lean_Elab_Term_elabSubst___lambda__6___closed__8 = _init_l_Lean_Elab_Term_elabSubst___lambda__6___closed__8(); +lean_mark_persistent(l_Lean_Elab_Term_elabSubst___lambda__6___closed__8); +l_Lean_Elab_Term_elabSubst___lambda__6___closed__9 = _init_l_Lean_Elab_Term_elabSubst___lambda__6___closed__9(); +lean_mark_persistent(l_Lean_Elab_Term_elabSubst___lambda__6___closed__9); l_Lean_Elab_Term_elabSubst___closed__1 = _init_l_Lean_Elab_Term_elabSubst___closed__1(); lean_mark_persistent(l_Lean_Elab_Term_elabSubst___closed__1); l_Lean_Elab_Term_elabSubst___closed__2 = _init_l_Lean_Elab_Term_elabSubst___closed__2(); diff --git a/stage0/stdlib/Lean/Elab/Command.c b/stage0/stdlib/Lean/Elab/Command.c index dee76e855a04..9a71cc56f32a 100644 --- a/stage0/stdlib/Lean/Elab/Command.c +++ b/stage0/stdlib/Lean/Elab/Command.c @@ -15,7 +15,6 @@ extern "C" { #endif 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_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Command_0__Lean_Elab_Command_runCore___spec__4(lean_object*, size_t, size_t, lean_object*); -lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__12___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_getBracketedBinderIds___closed__9; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__16(lean_object*, lean_object*, size_t, size_t, lean_object*); @@ -30,20 +29,18 @@ static lean_object* l_List_foldl___at_Lean_Elab_Command_instAddErrorMessageConte lean_object* lean_format_pretty(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_liftAttrM___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabCommand___spec__23___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Command_runLinters___spec__10___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_logException___at_Lean_Elab_Command_runLinters___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabCommand___spec__20___at_Lean_Elab_Command_elabCommand___spec__21___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instMonadMacroAdapterCommandElabM___closed__1; -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*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadQuotationCommandElabM___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoTree___at_Lean_Elab_Command_expandDeclId___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__17(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_mkState___closed__6; 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_mkMessageAux___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instInhabitedScope___closed__2; -lean_object* l_Lean_MapDeclarationExtension_insert___rarg(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_instBEqOfDecidableEq___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_lintersRef; static lean_object* l_Lean_Elab_Command_getBracketedBinderIds___closed__5; @@ -59,34 +56,31 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Comma LEAN_EXPORT lean_object* l_Lean_Elab_addCompletionInfo___at_Lean_withSetOptionIn___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); static lean_object* l_Lean_Elab_elabSetOption___at_Lean_withSetOptionIn___spec__1___closed__4; -static lean_object* l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9___closed__2; static lean_object* l_Lean_Elab_Command_liftTermElabM___rarg___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Command_liftTermElabM(lean_object*); static lean_object* l_Lean_Elab_Command_instMonadRecDepthCommandElabM___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_isIncrementalElab___at___private_Lean_Elab_Command_0__Lean_Elab_Command_elabCommandUsing___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_CommandContextInfo_save___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instMonadEnvCommandElabM___closed__3; -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*); static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_631____closed__10; static lean_object* l_Lean_Elab_isIncrementalElab___at___private_Lean_Elab_Command_0__Lean_Elab_Command_elabCommandUsing___spec__4___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___boxed(lean_object*, 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_Lean_addDocString_x27___at_Lean_Elab_Command_expandDeclId___spec__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); 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*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Language_instInhabitedDynamicSnapshot; static lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_elabCommandUsing___closed__1; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__3(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__18(lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Elab_Command_getBracketedBinderIds___closed__6; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___auto____x40_Lean_Elab_Command___hyg_456____closed__15; -static lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__1___closed__2; -lean_object* lean_private_to_user_name(lean_object*); LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Command_runLinters___spec__10___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_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_Lean_Elab_Command_runTermElabM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_liftTermElabM___spec__10(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_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_Array_forInUnsafe_loop___at_Lean_Elab_Command_runLinters___spec__9___lambda__2___closed__2; -static lean_object* l_Lean_liftCommandElabM___rarg___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_4859_(lean_object*); static lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___lambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_profileitM___at_Lean_Elab_Command_runLinters___spec__15(lean_object*); @@ -95,8 +89,6 @@ static lean_object* l_Lean_Elab_Command_instMonadCommandElabM___closed__3; lean_object* l_Lean_PersistentArray_toArray___rarg(lean_object*); lean_object* l_Lean_profileitIOUnsafe___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_mkState___closed__11; -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_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_instMonadInfoTreeCommandElabM___closed__1; static lean_object* l_Lean_Elab_Command_elabCommand___lambda__3___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadTraceCommandElabM; @@ -109,12 +101,10 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabCom lean_object* l_Lean_Language_DynamicSnapshot_toTyped_x3f___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instInhabitedScope___closed__3; static lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_runCore___rarg___closed__1; -lean_object* l_Lean_ConstantInfo_levelParams(lean_object*); static lean_object* l_Lean_Elab_Command_mkState___closed__10; lean_object* l_Lean_indentD(lean_object*); double lean_float_div(double, double); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCommand___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___auto____x40_Lean_Elab_Command___hyg_456____closed__1; lean_object* l_Lean_Elab_mkMessageCore(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); lean_object* lean_io_promise_new(lean_object*); @@ -133,15 +123,15 @@ LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_Elab_Command_runLinter LEAN_EXPORT lean_object* l_Lean_Elab_Command_addUnivLevel___lambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instMonadQuotationCommandElabM___closed__2; lean_object* l_Lean_FileMap_toPosition(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_expandDeclId___spec__17(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_joinSep(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_expandDeclId___at_Lean_Elab_Command_expandDeclId___spec__1___closed__1; size_t lean_uint64_to_usize(uint64_t); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Command_0__Lean_Elab_Command_mkTermContext___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_mkState___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_withSaveInfoContext___at_Lean_Elab_Command_liftTermElabM___spec__1(lean_object*); LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_Elab_Command_liftTermElabM___spec__13___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___auto____x40_Lean_Elab_Command___hyg_456____closed__12; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___lambda__2___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoLeaf___at_Lean_withSetOptionIn___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); 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_elabCommandTopLevel(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Command_0__Lean_Elab_Command_runCore___spec__3(lean_object*, size_t, size_t, lean_object*); @@ -149,13 +139,11 @@ LEAN_EXPORT lean_object* l_Lean_Elab_logException___at_Lean_Elab_Command_elabCom LEAN_EXPORT lean_object* l_Lean_PersistentArray_forInAux___at_Lean_Elab_Command_elabCommandTopLevel___spec__4___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*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabCommand___spec__25___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_addDocString___at_Lean_Elab_Command_expandDeclId___spec__14(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Command_runLinters___spec__10___lambda__4(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_withTraceNode___at_Lean_Elab_Command_runLinters___spec__4___lambda__3___closed__1; lean_object* l_Lean_Syntax_getId(lean_object*); static lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___lambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Elab_Command_elabCommandTopLevel___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_expandDeclId___spec__17___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_getScope___boxed(lean_object*); static lean_object* l_Lean_Elab_Command_instInhabitedCommandElabM___closed__2; lean_object* l_Lean_Expr_sort___override(lean_object*); @@ -169,26 +157,19 @@ static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_27 lean_object* l_Array_toSubarray___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_Elab_Command_liftTermElabM___spec__13(lean_object*); static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_631____closed__12; -lean_object* l_String_removeLeadingSpaces(lean_object*); lean_object* l_Array_qpartition___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_runLinters___spec__9___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadMacroAdapterCommandElabM___lambda__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_mkCommandElabAttributeUnsafe___closed__3; static lean_object* l_Lean_Elab_Command_runLinters___closed__1; -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__4___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_getScopes___boxed(lean_object*); lean_object* lean_mk_array(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_mkState___closed__9; lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Language_instInhabitedDynamicSnapshot___spec__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_4827____closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadInfoTreeCommandElabM___lambda__2(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_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_expandDeclId___at_Lean_Elab_Command_expandDeclId___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instMonadRecDepthCommandElabM___closed__4; LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_Elab_Command_runLinters___spec__8(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkState(lean_object*, lean_object*, lean_object*); @@ -209,7 +190,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCommand(lean_object*, lean_obje LEAN_EXPORT lean_object* l_Lean_Elab_Command_withoutCommandIncrementality___rarg___lambda__1___boxed(lean_object*, lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_liftCoreM___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__4___closed__2; LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapMAux___at___private_Lean_Elab_Command_0__Lean_Elab_Command_runCore___spec__2___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Command_0__Lean_Elab_Command_runCore___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); @@ -217,8 +197,6 @@ static lean_object* l_Lean_withSetOptionIn___closed__3; static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_631____closed__16; LEAN_EXPORT lean_object* l_Lean_Elab_Command_liftCoreM(lean_object*); lean_object* l_Lean_Syntax_getTailPos_x3f(lean_object*, uint8_t); -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_EXPORT lean_object* l_Lean_mkConstWithLevelParams___at_Lean_Elab_Command_expandDeclId___spec__8(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_getScopes___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Command_runLinters___spec__6(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCommand___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -232,10 +210,8 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Command LEAN_EXPORT lean_object* l_Array_qsort_sort___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__14(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*); 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*); -static lean_object* l_Lean_addDocString___at_Lean_Elab_Command_expandDeclId___spec__14___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__12___rarg(lean_object*); lean_object* l_Lean_Elab_InfoTree_format(lean_object*, lean_object*, lean_object*); -lean_object* lean_environment_find(lean_object*, lean_object*); uint8_t lean_float_decLt(double, double); LEAN_EXPORT lean_object* l_Lean_Elab_Command_addUnivLevel___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); @@ -244,6 +220,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_getResetTraces___at LEAN_EXPORT lean_object* l_Lean_Elab_Command_liftCoreM___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_runLinters___spec__9___lambda__1___closed__1; 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*); +static lean_object* l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___closed__1; lean_object* l_Lean_MessageData_hasSyntheticSorry(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_runLinters___spec__9___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_isIncrementalElab___at___private_Lean_Elab_Command_0__Lean_Elab_Command_elabCommandUsing___spec__4___closed__1; @@ -251,7 +228,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_getLevelNames(lean_object*); static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_631____closed__13; static lean_object* l_Lean_Elab_Command_elabCommand___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Command_runLinters___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -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*); 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*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_liftTermElabM___spec__11(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__11(lean_object*, lean_object*, lean_object*, lean_object*); @@ -259,9 +235,9 @@ extern lean_object* l_Lean_LocalContext_empty; LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_withSaveInfoContext___at_Lean_Elab_Command_liftTermElabM___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_Elab_Command_instMonadLogCommandElabM; +static lean_object* l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___closed__3; lean_object* lean_io_get_num_heartbeats(lean_object*); uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_expandDeclId___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_elabSetOption___at_Lean_withSetOptionIn___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Nat_nextPowerOfTwo_go(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabCommand___lambda__3___closed__4; @@ -288,14 +264,11 @@ LEAN_EXPORT lean_object* l_Lean_logAt___at_Lean_Elab_Command_runLinters___spec__ static lean_object* l_Lean_Elab_Command_instImpl____x40_Lean_Elab_Command___hyg_3614____closed__1; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_runLinters___spec__9___closed__1; extern lean_object* l_Lean_maxRecDepth; -LEAN_EXPORT lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabCommand___spec__20___closed__1; lean_object* l_Lean_KVMap_insertCore(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__3___closed__1; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__15___closed__3; lean_object* l_List_head_x21___rarg(lean_object*, lean_object*); lean_object* l_Lean_Elab_expandMacroImpl_x3f___boxed(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*); uint8_t lean_string_dec_eq(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_mkCommandElabAttributeUnsafe___closed__5; static lean_object* l___auto____x40_Lean_Elab_Command___hyg_456____closed__13; @@ -303,9 +276,8 @@ LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCo LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__17___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadExceptOfExceptionCommandElabM___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_forInAux___at_Lean_Elab_Command_elabCommandTopLevel___spec__4___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -uint8_t l_Lean_Name_isPrefixOf(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_EXPORT lean_object* l_Lean_liftCommandElabM___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_liftCommandElabM___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_instBEqProd___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_runCore___rarg___closed__5; static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_631____closed__7; @@ -317,11 +289,8 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadRecDepthCommandElabM___lam LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Command_runLinters___spec__10(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_Elab_Command_elabCommand___spec__26___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at_Lean_Elab_Command_liftTermElabM___spec__2___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_addDocString___at_Lean_Elab_Command_expandDeclId___spec__14___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Kernel_enableDiag(lean_object*, uint8_t); static lean_object* l_Lean_withTraceNode___at_Lean_Elab_Command_runLinters___spec__4___lambda__4___closed__3; -static lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___lambda__2___closed__1; -lean_object* l_List_mapTR_loop___at_Lean_mkConstWithLevelParams___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadResolveNameCommandElabM; static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_4786____closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_addCompletionInfo___at_Lean_withSetOptionIn___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -335,7 +304,6 @@ LEAN_EXPORT lean_object* l_Lean_logAt___at_Lean_Elab_Command_runLinters___spec__ LEAN_EXPORT lean_object* l_Lean_Elab_Command_withoutCommandIncrementality___rarg(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_foldl___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__2___closed__1; static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_4827____closed__2; -uint8_t l_Lean_isReservedName(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabCommand___lambda__6___closed__3; LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Command_runLinters___spec__4___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, 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__17(lean_object*, size_t, size_t, lean_object*); @@ -354,7 +322,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___h 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__10(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadInfoTreeCommandElabM___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__8; LEAN_EXPORT lean_object* l_Lean_PersistentArray_forIn___at_Lean_Elab_Command_elabCommandTopLevel___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_liftAttrM(lean_object*); lean_object* lean_io_promise_resolve(lean_object*, lean_object*, lean_object*); @@ -375,16 +342,14 @@ LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Command_runLinters_ LEAN_EXPORT lean_object* l_Lean_PersistentArray_forIn___at_Lean_Elab_Command_elabCommandTopLevel___spec__3___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___auto____x40_Lean_Elab_Command___hyg_456____closed__10; LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadRecDepthCommandElabM___lambda__2___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_liftCommandElabM___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_withSetOptionIn___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_liftTermElabM___rarg___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Command_0__Lean_Elab_Command_runCore___spec__5(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadEnvCommandElabM; -static lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__3___closed__2; uint8_t l_List_elem___at_Lean_addAliasEntry___spec__16(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_631_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCommand___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_mkCommandElabAttributeUnsafe___closed__4; -LEAN_EXPORT lean_object* l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___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; LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__17___rarg(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_getVarDecls___boxed(lean_object*); @@ -398,21 +363,19 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_commandElabAttribute; static lean_object* l_Lean_Elab_elabSetOption___at_Lean_withSetOptionIn___spec__1___closed__1; LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Command_runLinters___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_mkCommandElabAttributeUnsafe___closed__8; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___spec__1(lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* l_Lean_Elab_expandMacroImpl_x3f(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at_Lean_Elab_Command_liftTermElabM___spec__2___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_forInUnsafe_loop___at_Lean_Elab_Command_runLinters___spec__9___lambda__3(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_liftIO___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_getBracketedBinderIds(lean_object*, lean_object*, 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*); LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_Elab_Command_liftCoreM___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_ResolveName_resolveNamespace(lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_mkPrivateName(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_mkState___closed__12; LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Command_runLinters___spec__6___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__12___rarg___closed__1; -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__10(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_631____closed__1; uint64_t lean_uint64_shift_right(uint64_t, uint64_t); LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__17___boxed(lean_object*, lean_object*); @@ -425,9 +388,9 @@ lean_object* l_Lean_MessageData_ofSyntax(lean_object*); 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_EXPORT lean_object* l_Lean_Elab_Command_instMonadInfoTreeCommandElabM; LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadTraceCommandElabM___lambda__2(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_div(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCommand___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoTree___at_Lean_withSetOptionIn___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_liftIO(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Command_0__Lean_Elab_Command_mkTermContext___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadResolveNameCommandElabM___lambda__2(lean_object*, lean_object*, lean_object*); @@ -444,23 +407,22 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadLiftTIOCommandElabM(lean_o static lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_withSaveInfoContext___at_Lean_Elab_Command_liftTermElabM___spec__1___rarg___lambda__1(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__13(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_withSetOptionIn___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_mkCommandElabAttributeUnsafe___closed__7; static lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_runCore___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_getRef(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore(lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_withSetOptionIn___spec__7___boxed(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*); lean_object* l_Lean_throwError___at_Lean_realizeGlobalConstCore___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instMonadQuotationCommandElabM___closed__1; static lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___lambda__1___closed__7; LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadResolveNameCommandElabM___lambda__1___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__3; -static lean_object* l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadMacroAdapterCommandElabM___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___auto____x40_Lean_Elab_Command___hyg_456____closed__18; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_liftTermElabM___spec__7(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___lambda__2___closed__2; 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_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___auto____x40_Lean_Elab_Command___hyg_456_; lean_object* l_Lean_Syntax_getKind(lean_object*); static lean_object* l_Lean_withSetOptionIn___closed__1; @@ -479,26 +441,22 @@ LEAN_EXPORT lean_object* l_Lean_liftCommandElabM(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_runLinters___spec__9___lambda__2___closed__4; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_liftTermElabM___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_object* l_Lean_Meta_MetaM_run___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__3___boxed(lean_object*, lean_object*, 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(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCommand___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__19___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__5___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__6(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadEnvCommandElabM___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_runCore___rarg___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Command_liftTermElabM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Name_replacePrefix(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_getBracketedBinderIds___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_withScope(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabCommand___spec__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__16(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_runLinters___closed__2; static lean_object* l_Lean_Elab_logException___at_Lean_Elab_Command_runLinters___spec__1___closed__4; lean_object* lean_st_ref_get(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadLogCommandElabM___lambda__5(lean_object*, lean_object*, lean_object*, 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*); static lean_object* l_Lean_Elab_Command_mkState___closed__5; -LEAN_EXPORT lean_object* l_Lean_liftCommandElabM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_liftCommandElabM___rarg(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__12___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_Command_instMonadEnvCommandElabM___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadEvalTermElabMCommandElabM___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -511,7 +469,6 @@ static lean_object* l_Lean_Elab_Command_runLinters___lambda__1___closed__2; lean_object* lean_array_to_list(lean_object*); lean_object* l_ReaderT_instApplicativeOfMonad___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapM___at_Lean_Elab_Command_liftTermElabM___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_addDocString___at_Lean_Elab_Command_expandDeclId___spec__14___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_631____closed__14; static lean_object* l_Lean_Elab_Command_instMonadExceptOfExceptionCommandElabM___closed__1; LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -520,10 +477,9 @@ LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapMAux___at_Lean_Elab_Command_l LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_Elab_Command_runLinters___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); static lean_object* l_Lean_withTraceNode___at_Lean_Elab_Command_runLinters___spec__4___lambda__4___closed__2; -lean_object* l_Lean_Name_append(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_withSetOptionIn___closed__4; static lean_object* l_Lean_Elab_Command_instMonadTraceCommandElabM___closed__1; -static lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___closed__2; static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_631____closed__17; static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_4827____closed__5; LEAN_EXPORT lean_object* l_Lean_PersistentArray_forIn___at_Lean_Elab_Command_elabCommandTopLevel___spec__3___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -539,30 +495,26 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_modifyScope(lean_object*, lean_obje lean_object* l_Lean_Elab_InfoTree_substitute(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_getInfoTrees___at_Lean_Elab_Command_elabCommandTopLevel___spec__1___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_liftTermElabM___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_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5(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_Command_runLinters___spec__9___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_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__2___closed__1; lean_object* l_Lean_RBNode_insert___at_Lean_NameMap_insert___spec__1___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_getCurrMacroScope(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instMonadRefCommandElabM___closed__1; static lean_object* l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1___closed__2; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabCommand___spec__20___at_Lean_Elab_Command_elabCommand___spec__21___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoTree___at_Lean_withSetOptionIn___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_getMainModule___rarg___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_mkState___closed__2; -lean_object* l_Lean_Elab_expandDeclIdCore(lean_object*); +lean_object* lean_thunk_get_own(lean_object*); extern lean_object* l_Lean_Elab_builtinIncrementalElabs; static lean_object* l_Lean_Elab_Command_getBracketedBinderIds___closed__7; LEAN_EXPORT lean_object* l_Lean_profileitM___at_Lean_Elab_Command_runLinters___spec__15___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_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*); LEAN_EXPORT lean_object* l_Array_zipWithAux___at_Lean_Elab_Command_elabCommand___spec__18___boxed(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__2; static lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___lambda__1___closed__5; static lean_object* l_Lean_Elab_Command_instInhabitedScope___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__11___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_Command_initFn____x40_Lean_Elab_Command___hyg_631____closed__15; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__15(lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l___auto____x40_Lean_Elab_Command___hyg_456____closed__2; -lean_object* l_Lean_extractMacroScopes(lean_object*); static lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1___closed__3; static lean_object* l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_withMacroExpansion___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -570,7 +522,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_getResetTraces___at lean_object* l_instHashableProd___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadCommandElabM; LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadMacroAdapterCommandElabM___lambda__1(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__4___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); 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*); uint8_t lean_name_eq(lean_object*, lean_object*); static lean_object* l_Lean_withTraceNode___at_Lean_Elab_Command_runLinters___spec__4___lambda__4___closed__1; @@ -578,38 +529,37 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadEnvCommandElabM___lambda__ lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instMonadExceptOfExceptionCommandElabM___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_getBracketedBinderIds___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__18___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabCommand___spec__24(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCommand___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_warningAsError; extern lean_object* l_Lean_Elab_pp_macroStack; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___lambda__2(lean_object*); static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_getBracketedBinderIds___spec__1___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_mkState___closed__7; uint8_t l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_631____closed__4; -extern lean_object* l_Lean_docStringExt; +static lean_object* l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadExceptOfExceptionCommandElabM; 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_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCommandTopLevel___lambda__2___boxed(lean_object*); static lean_object* l_Lean_Elab_Command_mkCommandElabAttributeUnsafe___closed__1; extern lean_object* l_Lean_trace_profiler_threshold; LEAN_EXPORT 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_liftCommandElabM___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabCommand___spec__14___boxed(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_Command_instMonadQuotationCommandElabM; lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instMonadQuotationCommandElabM___closed__4; -static lean_object* l_Lean_liftCommandElabM___rarg___closed__2; static lean_object* l_Lean_Elab_Command_mkState___closed__1; uint8_t l_Lean_Syntax_matchesNull(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_liftCommandElabM___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instToSnapshotTreeMacroExpandedSnapshot(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_getMainModule___boxed(lean_object*); static lean_object* l_Lean_Elab_Command_modifyScope___closed__3; -static lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___closed__3; static lean_object* l_Lean_Elab_Command_modifyScope___closed__4; static lean_object* l_Lean_Elab_Command_liftTermElabM___rarg___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -628,22 +578,17 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_instTypeNameMacroExpandedSnapshot; LEAN_EXPORT lean_object* l_List_forM___at_Lean_Elab_Command_elabCommand___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadExceptOfExceptionCommandElabM___lambda__2(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_ioErrorToMessage(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___closed__1; LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_Elab_Command_liftCoreM___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Command_runLinters___spec__10___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_liftTermElabM___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_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_instToSnapshotTreeMacroExpandedSnapshot___spec__1___lambda__1___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadLogCommandElabM___lambda__2(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_addDocString_x27___at_Lean_Elab_Command_expandDeclId___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_withSetOptionIn___lambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_withLoggingExceptions(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabCommand___closed__7; lean_object* lean_task_get_own(lean_object*); static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_631____closed__6; extern lean_object* l_Std_Format_defWidth; -LEAN_EXPORT lean_object* l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_expandDeclId___spec__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_MacroScopesView_review(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_expandDeclId___at_Lean_Elab_Command_expandDeclId___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_mkElabAttribute___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___auto____x40_Lean_Elab_Command___hyg_456____closed__21; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); @@ -655,17 +600,17 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_liftTermE LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadLogCommandElabM___lambda__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instMonadMacroAdapterCommandElabM___closed__3; +LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Elab_Command_elabCommand___spec__19___lambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_addLinter(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instInhabitedCommandElabM___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_4786____closed__2; LEAN_EXPORT lean_object* l_Lean_PersistentArray_forInAux___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__9___lambda__1___boxed(lean_object*, lean_object*); +lean_object* lean_mk_thunk(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__15___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Command_runTermElabM___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Environment_contains(lean_object*, lean_object*); extern lean_object* l_Lean_inheritedTraceOptions; -lean_object* l_Lean_MessageData_ofExpr(lean_object*); 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_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_Command_initFn____x40_Lean_Elab_Command___hyg_4859____closed__1; @@ -683,7 +628,6 @@ static lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceA static lean_object* l_Lean_Elab_Command_elabCommand___lambda__6___closed__2; static lean_object* l_Lean_Elab_Command_instMonadCommandElabM___closed__6; static lean_object* l_Lean_Elab_Command_modifyScope___closed__2; -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* l_Lean_Elab_Term_withAutoBoundImplicit___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCommandTopLevel___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); @@ -698,7 +642,6 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Comma static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_3514____closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_liftTermElabM___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabCommand___spec__15(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*); extern lean_object* l_Lean_Core_interruptExceptionId; LEAN_EXPORT lean_object* l_Lean_Elab_Command_withFreshMacroScope___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabCommandTopLevel___lambda__3___closed__2; @@ -713,7 +656,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_addT LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_instToSnapshotTreeMacroExpandedSnapshot___spec__1(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_elabSetOption___at_Lean_withSetOptionIn___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_withoutCommandIncrementality___rarg___closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoTree___at_Lean_Elab_Command_expandDeclId___spec__12(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Command_runLinters___spec__4___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_logException___at_Lean_Elab_Command_elabCommand___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_3514____closed__2; @@ -727,17 +669,16 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_getScopes(lean_object*); static lean_object* l___auto____x40_Lean_Elab_Command___hyg_456____closed__4; lean_object* l_Lean_Syntax_setArgs(lean_object*, lean_object*); extern lean_object* l_Lean_NameSet_empty; +LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Elab_Command_elabCommand___spec__19___lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadOptionsCommandElabM___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Command_runLinters___spec__6___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCommand___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___auto____x40_Lean_Elab_Command___hyg_456____closed__19; LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Command_runLinters___spec__12___boxed(lean_object*); 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*); -uint8_t l_Lean_Name_isAtomic(lean_object*); LEAN_EXPORT lean_object* l_Lean_profileitM___at_Lean_Elab_Command_runLinters___spec__15___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_withInfoTreeContext___at___private_Lean_Elab_Command_0__Lean_Elab_Command_elabCommandUsing___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_runCore___rarg___closed__3; -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*); static lean_object* l_Lean_Elab_logException___at_Lean_Elab_Command_runLinters___spec__1___closed__3; static lean_object* l_Lean_Elab_Command_instAddMessageContextCommandElabM___closed__1; uint8_t lean_nat_dec_eq(lean_object*, lean_object*); @@ -754,7 +695,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadLogCommandElabM___lambda__ uint8_t lean_nat_dec_lt(lean_object*, lean_object*); lean_object* lean_environment_main_module(lean_object*); static lean_object* l_Lean_Elab_Command_liftTermElabM___rarg___closed__4; -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_withSetOptionIn___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_withInfoTreeContext___at_Lean_Elab_Command_withMacroExpansion___spec__1(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_Command_instMonadResolveNameCommandElabM___lambda__2___boxed(lean_object*, lean_object*, lean_object*); @@ -770,7 +710,6 @@ lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_isTracingEnabledFor___at_Lean_Elab_Command_runLinters___spec__11(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_631____closed__8; 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_addDocString___at_Lean_Elab_Command_expandDeclId___spec__14___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_withMacroExpansion___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_withFreshMacroScope(lean_object*); @@ -779,34 +718,26 @@ LEAN_EXPORT lean_object* l_Array_qsort_sort___at___private_Lean_Elab_Command_0__ LEAN_EXPORT lean_object* l_Lean_Elab_Command_getMainModule(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapM___at___private_Lean_Elab_Command_0__Lean_Elab_Command_runCore___spec__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forM___at_Lean_Elab_Command_elabCommand___spec__8(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_598_(lean_object*); -static lean_object* l_Lean_addDocString___at_Lean_Elab_Command_expandDeclId___spec__14___closed__1; +LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_liftCommandElabM___spec__1(lean_object*); static lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_elabCommandUsing___closed__2; static lean_object* l_Lean_Elab_Command_getBracketedBinderIds___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_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instMonadRefCommandElabM___closed__3; static lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___lambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadTraceCommandElabM___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_TagDeclarationExtension_tag(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_findAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__4___closed__1; LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Command_runLinters___spec__10___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadLogCommandElabM___lambda__3___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_runCore___rarg___lambda__1(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_NameSet_contains(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Option_get_x3f___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessages___spec__1___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_addDocString___at_Lean_Elab_Command_expandDeclId___spec__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_getBracketedBinderIds___spec__2___boxed(lean_object*, lean_object*, lean_object*); lean_object* lean_io_get_task_state(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instMonadInfoTreeCommandElabM___closed__2; uint8_t l_Lean_KVMap_getBool(lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapMAux___at_Lean_Elab_Command_liftTermElabM___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_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__2___boxed(lean_object*, lean_object*); uint64_t lean_uint64_xor(uint64_t, uint64_t); LEAN_EXPORT lean_object* l_Lean_Elab_Command_getScopes___rarg___boxed(lean_object*, lean_object*); @@ -820,7 +751,6 @@ lean_object* lean_panic_fn(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_getBracketedBinderIds___spec__1(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_Lean_throwError___at___private_Lean_Elab_Command_0__Lean_Elab_Command_elabCommandUsing___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___closed__2; static lean_object* l_Lean_withTraceNode___at_Lean_Elab_Command_runLinters___spec__4___lambda__2___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadEnvCommandElabM___lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadEnvCommandElabM___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); @@ -838,7 +768,6 @@ static lean_object* l___auto____x40_Lean_Elab_Command___hyg_456____closed__28; static lean_object* l_Lean_Elab_Command_withoutCommandIncrementality___rarg___closed__4; static lean_object* l_Array_qsort_sort___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__14___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_getInfoTrees___at_Lean_Elab_Command_elabCommandTopLevel___spec__1___rarg(lean_object*, lean_object*); -uint8_t l_Lean_isStructure(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at_Lean_Elab_Command_liftTermElabM___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCommand___lambda__7___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabCommand___spec__25(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); @@ -846,7 +775,6 @@ static double l_Lean_withTraceNode___at_Lean_Elab_Command_runLinters___spec__4__ LEAN_EXPORT lean_object* l_Lean_Elab_Command_liftCoreM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_mul(lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__15___closed__1; -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__19___closed__1; static lean_object* l___auto____x40_Lean_Elab_Command___hyg_456____closed__8; lean_object* l_Lean_Core_resetMessageLog(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_withSaveInfoContext___at_Lean_Elab_Command_liftTermElabM___spec__1___rarg___closed__1; @@ -857,14 +785,12 @@ static lean_object* l_Lean_Elab_logException___at_Lean_Elab_Command_runLinters__ lean_object* l_Lean_Elab_Term_withoutAutoBoundImplicit___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_DataValue_sameCtor(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_runLinters___spec__9___lambda__3___boxed(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_expandDeclId___spec__15(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Command_runLinters___spec__4___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabCommand___spec__20___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Command_instInhabitedCommandElabM(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_getInfoTrees___at_Lean_Elab_Command_elabCommandTopLevel___spec__1(lean_object*); lean_object* l_List_iotaTR(lean_object*); lean_object* l_Lean_Kernel_resetDiag___lambda__1(lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__19___closed__2; LEAN_EXPORT lean_object* l_Lean_PersistentArray_forIn___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabCommandTopLevel___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at_Lean_Elab_Command_liftTermElabM___spec__2(lean_object*); @@ -880,15 +806,12 @@ LEAN_EXPORT lean_object* l_Lean_PersistentArray_forIn___at_Lean_Elab_Command_ela static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_631____closed__9; 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_Command_initFn____x40_Lean_Elab_Command___hyg_4827_(lean_object*); -lean_object* l_Lean_Environment_getModuleIdxFor_x3f(lean_object*, lean_object*); -extern lean_object* l_Lean_protectedExt; -LEAN_EXPORT lean_object* l_Lean_mkConstWithLevelParams___at_Lean_Elab_Command_expandDeclId___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___auto____x40_Lean_Elab_Command___hyg_456____closed__11; static lean_object* l_Lean_Elab_Command_elabCommandTopLevel___lambda__3___closed__1; lean_object* lean_erase_macro_scopes(lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__18(lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Elab_incrementalAttr; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabCommand___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_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___lambda__1___boxed(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_Command___hyg_4827____closed__4; static lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___lambda__1___closed__9; lean_object* l_List_reverse___rarg(lean_object*); @@ -909,17 +832,13 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_runTermElabM___rarg___lambda__2___b LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadEvalTermElabMCommandElabM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabCommand___spec__24___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_instMonadRecDepthCommandElabM; -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__7; uint8_t l_Lean_Syntax_hasMissing(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_631____closed__11; size_t lean_usize_add(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadLogCommandElabM___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_addTraceNode___at_Lean_Elab_Command_runLinters___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabCommand___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandDeclId(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__12(lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__5; lean_object* l_Lean_Language_SnapshotTask_map___rarg(lean_object*, lean_object*, lean_object*, uint8_t); lean_object* l_Lean_MessageLog_append(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_ioErrorToMessage___boxed(lean_object*, lean_object*, lean_object*); @@ -934,11 +853,12 @@ uint8_t l_Lean_PersistentArray_isEmpty___rarg(lean_object*); lean_object* l_Lean_Language_SnapshotTask_get___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_forIn___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instMonadCommandElabM___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoLeaf___at_Lean_withSetOptionIn___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Language_SnapshotTree_trace(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_io_error_to_string(lean_object*); lean_object* l_Lean_KeyedDeclsAttribute_getEntries___rarg(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_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_withoutCommandIncrementality___rarg___lambda__2___boxed(lean_object*, lean_object*); lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); static lean_object* l___auto____x40_Lean_Elab_Command___hyg_456____closed__14; @@ -954,7 +874,6 @@ LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Command_runLinters_ static lean_object* l_Lean_Elab_Command_withoutCommandIncrementality___rarg___closed__1; static lean_object* l_Lean_Elab_Command_instMonadRecDepthCommandElabM___closed__3; LEAN_EXPORT lean_object* l_Lean_PersistentArray_forIn___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__8___lambda__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_liftCommandElabM___spec__1(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_getInfoTrees___at_Lean_Elab_Command_elabCommandTopLevel___spec__1___boxed(lean_object*); lean_object* lean_string_append(lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_runLinters___spec__9___lambda__2___closed__3; @@ -963,9 +882,7 @@ static lean_object* l___auto____x40_Lean_Elab_Command___hyg_456____closed__9; extern lean_object* l_Lean_trace_profiler_output; static lean_object* l_Lean_Elab_Command_withoutCommandIncrementality___rarg___closed__2; static lean_object* l_Lean_Elab_Command_instMonadTraceCommandElabM___closed__3; -lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Syntax_SepArray_getElems___spec__1(lean_object*, size_t, size_t, lean_object*); lean_object* lean_array_get_size(lean_object*); -static lean_object* l_Lean_liftCommandElabM___rarg___closed__3; LEAN_EXPORT lean_object* l_Lean_PersistentArray_forInAux___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_3514_(lean_object*); static lean_object* l_Lean_Elab_Command_runTermElabM___rarg___lambda__2___closed__1; @@ -975,42 +892,36 @@ LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabComma 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_PersistentArray_mapM___at___private_Lean_Elab_Command_0__Lean_Elab_Command_runCore___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_showPartialSyntaxErrors; -LEAN_EXPORT lean_object* l_Lean_Elab_checkIfShadowingStructureField___at_Lean_Elab_Command_expandDeclId___spec__3(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*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); 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*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadInfoTreeCommandElabM___lambda__1___boxed(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_EXPORT lean_object* l_Lean_Elab_Command_instMonadRefCommandElabM; lean_object* l_instHashablePos___boxed(lean_object*); extern lean_object* l_Lean_Elab_unsupportedSyntaxExceptionId; lean_object* l_Lean_MessageLog_toArray(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_EXPORT lean_object* l_Lean_Elab_Command_withMacroExpansion(lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_instToSnapshotTreeMacroExpandedSnapshot___spec__1___closed__1; static lean_object* l_Lean_Elab_Command_instMonadTraceCommandElabM___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_getBracketedBinderIds___spec__1___rarg(lean_object*); static lean_object* l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_addUnivLevel___spec__1___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandDeclId___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_mkCommandElabAttributeUnsafe___closed__2; +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_withSetOptionIn___spec__7(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__13___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_withoutCommandIncrementality(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_getBracketedBinderIds___spec__2(size_t, size_t, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_Command_withoutCommandIncrementality___rarg___lambda__1(uint8_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_addTraceNode___at_Lean_Elab_Command_runLinters___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__4; static lean_object* l_Lean_Elab_Command_modifyScope___closed__1; static lean_object* l_Lean_Elab_Command_instMonadResolveNameCommandElabM___closed__1; uint8_t l_Lean_Exception_isRuntime(lean_object*); LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Elab_Command_elabCommandTopLevel___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_qsort_sort___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__14___lambda__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_liftCommandElabM___rarg___lambda__1___boxed(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_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabCommandTopLevel___spec__6(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_addTraceNode___at_Lean_Elab_Command_runLinters___spec__13(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_expandDeclId___spec__19(lean_object*, 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_Command_liftTermElabM___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*); static lean_object* l_Lean_Elab_Command_instMonadMacroAdapterCommandElabM___closed__2; LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__16(lean_object*, lean_object*, lean_object*, lean_object*); @@ -1019,17 +930,15 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadInfoTreeCommandElabM___lam LEAN_EXPORT lean_object* l_Lean_log___at_Lean_Elab_Command_runLinters___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_getD___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1___closed__1; -lean_object* l_Lean_getStructureFieldsFlattened(lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instAddMessageContextCommandElabM; -LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_expandDeclId___spec__11(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_modifyScope___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_addUnivLevel___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabCommand___lambda__6___closed__4; static lean_object* l_Lean_Elab_Command_getBracketedBinderIds___closed__4; static lean_object* l_Lean_Elab_Command_getBracketedBinderIds___closed__10; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_runTermElabM___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_mkTermContext___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCommand___lambda__5(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_mkMetaContext___closed__1; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); @@ -1039,11 +948,9 @@ static lean_object* l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab lean_object* lean_dbg_trace(lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofName(lean_object*); LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Command_runLinters___spec__10___lambda__2(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, double, double, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__1; +LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_liftCommandElabM___spec__1___rarg(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*); static lean_object* l___auto____x40_Lean_Elab_Command___hyg_456____closed__23; -static lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___closed__4; -LEAN_EXPORT lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_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*); uint8_t l___private_Lean_Message_0__Lean_beqMessageSeverity____x40_Lean_Message___hyg_106_(uint8_t, uint8_t); LEAN_EXPORT lean_object* l_Lean_Elab_Command_withoutCommandIncrementality___rarg___lambda__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadRecDepthCommandElabM___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1060,10 +967,10 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadRecDepthCommandElabM___lam LEAN_EXPORT lean_object* l_Lean_Elab_Command_liftTermElabM___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_isTracingEnabledFor___at_Lean_Elab_Command_runLinters___spec__11___boxed(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_throwError___at_Lean_withSetOptionIn___spec__5(lean_object*, lean_object*, lean_object*, lean_object*); double lean_float_sub(double, double); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadExceptOfExceptionCommandElabM___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_liftCommandElabM___rarg___lambda__1(lean_object*); -LEAN_EXPORT lean_object* l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_liftCommandElabM___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_liftTermElabM___rarg___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_getVarDecls(lean_object*); uint8_t l_Array_isEmpty___rarg(lean_object*); @@ -18992,10 +18899,10 @@ return x_1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_instToSnapshotTreeMacroExpandedSnapshot___spec__1___lambda__1(lean_object* x_1) { _start: { -lean_object* x_2; +lean_object* x_2; lean_object* x_3; x_2 = lean_ctor_get(x_1, 1); -lean_inc(x_2); -return x_2; +x_3 = lean_thunk_get_own(x_2); +return x_3; } } static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Elab_Command_instToSnapshotTreeMacroExpandedSnapshot___spec__1___closed__1() { @@ -21755,29 +21662,39 @@ goto _start; } } } +LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Elab_Command_elabCommand___spec__19___lambda__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; size_t x_5; size_t x_6; lean_object* x_7; lean_object* x_8; +x_3 = lean_ctor_get(x_1, 0); +lean_inc(x_3); +x_4 = lean_ctor_get(x_1, 4); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_array_size(x_4); +x_6 = 0; +x_7 = l_Array_mapMUnsafe_map___at_Lean_Elab_Command_instToSnapshotTreeMacroExpandedSnapshot___spec__1(x_5, x_6, x_4); +x_8 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_8, 0, x_3); +lean_ctor_set(x_8, 1, x_7); +return x_8; +} +} LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Elab_Command_elabCommand___spec__19(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_3; lean_object* x_4; lean_object* x_5; size_t x_6; size_t x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_inc(x_2); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); -x_4 = lean_ctor_get(x_2, 0); -lean_inc(x_4); -x_5 = lean_ctor_get(x_2, 4); -lean_inc(x_5); -lean_dec(x_2); -x_6 = lean_array_size(x_5); -x_7 = 0; -x_8 = l_Array_mapMUnsafe_map___at_Lean_Elab_Command_instToSnapshotTreeMacroExpandedSnapshot___spec__1(x_6, x_7, x_5); -x_9 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_9, 0, x_4); -lean_ctor_set(x_9, 1, x_8); -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_3); -lean_ctor_set(x_10, 1, x_9); -return x_10; +x_4 = lean_alloc_closure((void*)(l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Elab_Command_elabCommand___spec__19___lambda__1___boxed), 2, 1); +lean_closure_set(x_4, 0, x_2); +x_5 = lean_mk_thunk(x_4); +x_6 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_6, 0, x_3); +lean_ctor_set(x_6, 1, x_5); +return x_6; } } static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabCommand___spec__20___closed__1() { @@ -26051,6 +25968,15 @@ lean_dec(x_1); return x_5; } } +LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Elab_Command_elabCommand___spec__19___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Elab_Command_elabCommand___spec__19___lambda__1(x_1, x_2); +lean_dec(x_2); +return x_3; +} +} LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabCommand___spec__20___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { @@ -27889,34 +27815,34 @@ x_23 = l_Lean_Syntax_hasMissing(x_1); x_24 = lean_st_ref_take(x_3, x_7); if (x_23 == 0) { -uint8_t x_293; +uint8_t x_339; lean_dec(x_11); -x_293 = 0; -x_25 = x_293; -goto block_292; +x_339 = 0; +x_25 = x_339; +goto block_338; } else { -lean_object* x_294; uint8_t x_295; -x_294 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__3___closed__2; -x_295 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_11, x_294); +lean_object* x_340; uint8_t x_341; +x_340 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__3___closed__2; +x_341 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_11, x_340); lean_dec(x_11); -if (x_295 == 0) +if (x_341 == 0) { -uint8_t x_296; -x_296 = 1; -x_25 = x_296; -goto block_292; +uint8_t x_342; +x_342 = 1; +x_25 = x_342; +goto block_338; } else { -uint8_t x_297; -x_297 = 0; -x_25 = x_297; -goto block_292; +uint8_t x_343; +x_343 = 0; +x_25 = x_343; +goto block_338; } } -block_292: +block_338: { lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; x_26 = lean_ctor_get(x_24, 0); @@ -27944,7 +27870,7 @@ lean_ctor_set_uint8(x_28, sizeof(void*)*10, x_25); x_29 = !lean_is_exclusive(x_26); if (x_29 == 0) { -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_92; lean_object* x_93; lean_object* x_147; +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_104; lean_object* x_105; lean_object* x_171; x_30 = lean_ctor_get(x_26, 1); x_31 = l___private_Lean_Elab_Command_0__Lean_Elab_Command_runCore___rarg___closed__4; lean_ctor_set(x_26, 1, x_31); @@ -27961,74 +27887,74 @@ lean_dec(x_34); lean_inc(x_3); lean_inc(x_28); lean_inc(x_1); -x_147 = l_Lean_Elab_Command_elabCommand(x_1, x_28, x_3, x_36); -if (lean_obj_tag(x_147) == 0) +x_171 = l_Lean_Elab_Command_elabCommand(x_1, x_28, x_3, x_36); +if (lean_obj_tag(x_171) == 0) { -lean_object* x_148; lean_object* x_149; lean_object* x_150; -x_148 = lean_ctor_get(x_147, 1); -lean_inc(x_148); -lean_dec(x_147); -x_149 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__3___closed__1; +lean_object* x_172; lean_object* x_173; lean_object* x_174; +x_172 = lean_ctor_get(x_171, 1); +lean_inc(x_172); +lean_dec(x_171); +x_173 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__3___closed__1; lean_inc(x_1); -x_150 = l_Lean_Syntax_findAux(x_149, x_1); -if (lean_obj_tag(x_150) == 0) +x_174 = l_Lean_Syntax_findAux(x_173, x_1); +if (lean_obj_tag(x_174) == 0) { -lean_object* x_151; lean_object* x_152; -x_151 = lean_alloc_closure((void*)(l_Lean_Elab_Command_runLinters), 4, 1); -lean_closure_set(x_151, 0, x_1); +lean_object* x_175; lean_object* x_176; +x_175 = lean_alloc_closure((void*)(l_Lean_Elab_Command_runLinters), 4, 1); +lean_closure_set(x_175, 0, x_1); lean_inc(x_3); lean_inc(x_28); -x_152 = l_Lean_Elab_withLogging___at_Lean_Elab_Command_elabCommand___spec__2(x_151, x_28, x_3, x_148); -if (lean_obj_tag(x_152) == 0) +x_176 = l_Lean_Elab_withLogging___at_Lean_Elab_Command_elabCommand___spec__2(x_175, x_28, x_3, x_172); +if (lean_obj_tag(x_176) == 0) { -lean_object* x_153; lean_object* x_154; -x_153 = lean_ctor_get(x_152, 0); -lean_inc(x_153); -x_154 = lean_ctor_get(x_152, 1); -lean_inc(x_154); -lean_dec(x_152); -x_37 = x_153; -x_38 = x_154; -goto block_91; +lean_object* x_177; lean_object* x_178; +x_177 = lean_ctor_get(x_176, 0); +lean_inc(x_177); +x_178 = lean_ctor_get(x_176, 1); +lean_inc(x_178); +lean_dec(x_176); +x_37 = x_177; +x_38 = x_178; +goto block_103; } else { -lean_object* x_155; lean_object* x_156; -x_155 = lean_ctor_get(x_152, 0); -lean_inc(x_155); -x_156 = lean_ctor_get(x_152, 1); -lean_inc(x_156); -lean_dec(x_152); -x_92 = x_155; -x_93 = x_156; -goto block_146; +lean_object* x_179; lean_object* x_180; +x_179 = lean_ctor_get(x_176, 0); +lean_inc(x_179); +x_180 = lean_ctor_get(x_176, 1); +lean_inc(x_180); +lean_dec(x_176); +x_104 = x_179; +x_105 = x_180; +goto block_170; } } else { -lean_object* x_157; -lean_dec(x_150); +lean_object* x_181; +lean_dec(x_174); lean_dec(x_1); -x_157 = lean_box(0); -x_37 = x_157; -x_38 = x_148; -goto block_91; +x_181 = lean_box(0); +x_37 = x_181; +x_38 = x_172; +goto block_103; } } else { -lean_object* x_158; lean_object* x_159; +lean_object* x_182; lean_object* x_183; lean_dec(x_1); -x_158 = lean_ctor_get(x_147, 0); -lean_inc(x_158); -x_159 = lean_ctor_get(x_147, 1); -lean_inc(x_159); -lean_dec(x_147); -x_92 = x_158; -x_93 = x_159; -goto block_146; +x_182 = lean_ctor_get(x_171, 0); +lean_inc(x_182); +x_183 = lean_ctor_get(x_171, 1); +lean_inc(x_183); +lean_dec(x_171); +x_104 = x_182; +x_105 = x_183; +goto block_170; } -block_91: +block_103: { lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; x_39 = lean_st_ref_get(x_3, x_38); @@ -28051,80 +27977,54 @@ x_47 = l_Lean_PersistentArray_forIn___at_Lean_Elab_Command_elabCommandTopLevel__ lean_dec(x_44); if (lean_obj_tag(x_47) == 0) { -if (lean_obj_tag(x_20) == 0) -{ -lean_object* x_48; lean_object* x_49; uint8_t x_50; +lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; uint8_t x_52; x_48 = lean_ctor_get(x_47, 1); lean_inc(x_48); lean_dec(x_47); -x_49 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_30, x_42, x_35, x_46, x_28, x_3, x_48); -lean_dec(x_3); -x_50 = !lean_is_exclusive(x_49); -if (x_50 == 0) -{ -lean_object* x_51; -x_51 = lean_ctor_get(x_49, 0); +x_49 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_4859____closed__5; +x_50 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Command_runLinters___spec__11(x_49, x_28, x_3, x_48); +x_51 = lean_ctor_get(x_50, 0); +lean_inc(x_51); +x_52 = lean_unbox(x_51); lean_dec(x_51); -lean_ctor_set(x_49, 0, x_37); -return x_49; -} -else -{ -lean_object* x_52; lean_object* x_53; -x_52 = lean_ctor_get(x_49, 1); -lean_inc(x_52); -lean_dec(x_49); -x_53 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_53, 0, x_37); -lean_ctor_set(x_53, 1, x_52); -return x_53; -} -} -else +if (x_52 == 0) { -lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; uint8_t x_58; lean_object* x_59; lean_object* x_81; lean_object* x_82; -x_54 = lean_ctor_get(x_47, 1); -lean_inc(x_54); -lean_dec(x_47); -x_55 = lean_ctor_get(x_20, 0); -lean_inc(x_55); +lean_object* x_53; lean_object* x_54; uint8_t x_55; lean_dec(x_20); -x_56 = lean_ctor_get(x_55, 1); -lean_inc(x_56); -lean_dec(x_55); -x_57 = lean_io_promise_result(x_56); -x_81 = lean_io_get_task_state(x_57, x_54); -x_82 = lean_ctor_get(x_81, 0); -lean_inc(x_82); -if (lean_obj_tag(x_82) == 2) +x_53 = lean_ctor_get(x_50, 1); +lean_inc(x_53); +lean_dec(x_50); +x_54 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_30, x_42, x_35, x_46, x_28, x_3, x_53); +lean_dec(x_3); +x_55 = !lean_is_exclusive(x_54); +if (x_55 == 0) { -lean_object* x_83; uint8_t x_84; -x_83 = lean_ctor_get(x_81, 1); -lean_inc(x_83); -lean_dec(x_81); -x_84 = 1; -x_58 = x_84; -x_59 = x_83; -goto block_80; +lean_object* x_56; +x_56 = lean_ctor_get(x_54, 0); +lean_dec(x_56); +lean_ctor_set(x_54, 0, x_37); +return x_54; } else { -lean_object* x_85; uint8_t x_86; -lean_dec(x_82); -x_85 = lean_ctor_get(x_81, 1); -lean_inc(x_85); -lean_dec(x_81); -x_86 = 0; -x_58 = x_86; -x_59 = x_85; -goto block_80; +lean_object* x_57; lean_object* x_58; +x_57 = lean_ctor_get(x_54, 1); +lean_inc(x_57); +lean_dec(x_54); +x_58 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_58, 0, x_37); +lean_ctor_set(x_58, 1, x_57); +return x_58; } -block_80: +} +else { -if (x_58 == 0) +if (lean_obj_tag(x_20) == 0) { -lean_object* x_60; uint8_t x_61; -lean_dec(x_57); +lean_object* x_59; lean_object* x_60; uint8_t x_61; +x_59 = lean_ctor_get(x_50, 1); +lean_inc(x_59); +lean_dec(x_50); x_60 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_30, x_42, x_35, x_46, x_28, x_3, x_59); lean_dec(x_3); x_61 = !lean_is_exclusive(x_60); @@ -28150,25 +28050,51 @@ return x_64; } else { -lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_65 = lean_task_get_own(x_57); -x_66 = lean_ctor_get(x_65, 1); +lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; uint8_t x_69; lean_object* x_70; lean_object* x_93; lean_object* x_94; +x_65 = lean_ctor_get(x_50, 1); +lean_inc(x_65); +lean_dec(x_50); +x_66 = lean_ctor_get(x_20, 0); lean_inc(x_66); -lean_dec(x_65); -x_67 = lean_alloc_closure((void*)(l_Lean_Language_SnapshotTree_trace), 4, 1); -lean_closure_set(x_67, 0, x_66); -x_68 = l_Lean_Elab_Command_liftCoreM___rarg(x_67, x_28, x_3, x_59); -if (lean_obj_tag(x_68) == 0) +lean_dec(x_20); +x_67 = lean_ctor_get(x_66, 1); +lean_inc(x_67); +lean_dec(x_66); +x_68 = lean_io_promise_result(x_67); +x_93 = lean_io_get_task_state(x_68, x_65); +x_94 = lean_ctor_get(x_93, 0); +lean_inc(x_94); +if (lean_obj_tag(x_94) == 2) { -lean_object* x_69; lean_object* x_70; lean_object* x_71; uint8_t x_72; -x_69 = lean_ctor_get(x_68, 0); -lean_inc(x_69); -x_70 = lean_ctor_get(x_68, 1); -lean_inc(x_70); +lean_object* x_95; uint8_t x_96; +x_95 = lean_ctor_get(x_93, 1); +lean_inc(x_95); +lean_dec(x_93); +x_96 = 1; +x_69 = x_96; +x_70 = x_95; +goto block_92; +} +else +{ +lean_object* x_97; uint8_t x_98; +lean_dec(x_94); +x_97 = lean_ctor_get(x_93, 1); +lean_inc(x_97); +lean_dec(x_93); +x_98 = 0; +x_69 = x_98; +x_70 = x_97; +goto block_92; +} +block_92: +{ +if (x_69 == 0) +{ +lean_object* x_71; uint8_t x_72; lean_dec(x_68); -x_71 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_30, x_42, x_35, x_69, x_28, x_3, x_70); +x_71 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_30, x_42, x_35, x_46, x_28, x_3, x_70); lean_dec(x_3); -lean_dec(x_69); x_72 = !lean_is_exclusive(x_71); if (x_72 == 0) { @@ -28192,30 +28118,75 @@ return x_75; } else { -uint8_t x_76; +lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; +x_76 = lean_task_get_own(x_68); +x_77 = lean_ctor_get(x_76, 1); +lean_inc(x_77); +lean_dec(x_76); +x_78 = lean_thunk_get_own(x_77); +lean_dec(x_77); +x_79 = lean_alloc_closure((void*)(l_Lean_Language_SnapshotTree_trace), 4, 1); +lean_closure_set(x_79, 0, x_78); +x_80 = l_Lean_Elab_Command_liftCoreM___rarg(x_79, x_28, x_3, x_70); +if (lean_obj_tag(x_80) == 0) +{ +lean_object* x_81; lean_object* x_82; lean_object* x_83; uint8_t x_84; +x_81 = lean_ctor_get(x_80, 0); +lean_inc(x_81); +x_82 = lean_ctor_get(x_80, 1); +lean_inc(x_82); +lean_dec(x_80); +x_83 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_30, x_42, x_35, x_81, x_28, x_3, x_82); +lean_dec(x_3); +lean_dec(x_81); +x_84 = !lean_is_exclusive(x_83); +if (x_84 == 0) +{ +lean_object* x_85; +x_85 = lean_ctor_get(x_83, 0); +lean_dec(x_85); +lean_ctor_set(x_83, 0, x_37); +return x_83; +} +else +{ +lean_object* x_86; lean_object* x_87; +x_86 = lean_ctor_get(x_83, 1); +lean_inc(x_86); +lean_dec(x_83); +x_87 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_87, 0, x_37); +lean_ctor_set(x_87, 1, x_86); +return x_87; +} +} +else +{ +uint8_t x_88; lean_dec(x_42); lean_dec(x_37); lean_dec(x_35); lean_dec(x_30); lean_dec(x_28); lean_dec(x_3); -x_76 = !lean_is_exclusive(x_68); -if (x_76 == 0) +x_88 = !lean_is_exclusive(x_80); +if (x_88 == 0) { -return x_68; +return x_80; } else { -lean_object* x_77; lean_object* x_78; lean_object* x_79; -x_77 = lean_ctor_get(x_68, 0); -x_78 = lean_ctor_get(x_68, 1); -lean_inc(x_78); -lean_inc(x_77); -lean_dec(x_68); -x_79 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_79, 0, x_77); -lean_ctor_set(x_79, 1, x_78); -return x_79; +lean_object* x_89; lean_object* x_90; lean_object* x_91; +x_89 = lean_ctor_get(x_80, 0); +x_90 = lean_ctor_get(x_80, 1); +lean_inc(x_90); +lean_inc(x_89); +lean_dec(x_80); +x_91 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_91, 0, x_89); +lean_ctor_set(x_91, 1, x_90); +return x_91; +} } } } @@ -28224,7 +28195,7 @@ return x_79; } else { -uint8_t x_87; +uint8_t x_99; lean_dec(x_42); lean_dec(x_37); lean_dec(x_35); @@ -28232,217 +28203,263 @@ lean_dec(x_30); lean_dec(x_28); lean_dec(x_20); lean_dec(x_3); -x_87 = !lean_is_exclusive(x_47); -if (x_87 == 0) +x_99 = !lean_is_exclusive(x_47); +if (x_99 == 0) { return x_47; } else { -lean_object* x_88; lean_object* x_89; lean_object* x_90; -x_88 = lean_ctor_get(x_47, 0); -x_89 = lean_ctor_get(x_47, 1); -lean_inc(x_89); -lean_inc(x_88); +lean_object* x_100; lean_object* x_101; lean_object* x_102; +x_100 = lean_ctor_get(x_47, 0); +x_101 = lean_ctor_get(x_47, 1); +lean_inc(x_101); +lean_inc(x_100); lean_dec(x_47); -x_90 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_90, 0, x_88); -lean_ctor_set(x_90, 1, x_89); -return x_90; +x_102 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_102, 0, x_100); +lean_ctor_set(x_102, 1, x_101); +return x_102; } } } -block_146: +block_170: { -lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; -x_94 = lean_st_ref_get(x_3, x_93); -x_95 = lean_ctor_get(x_94, 0); -lean_inc(x_95); -x_96 = lean_ctor_get(x_94, 1); -lean_inc(x_96); -lean_dec(x_94); -x_97 = lean_ctor_get(x_95, 1); -lean_inc(x_97); -lean_dec(x_95); -x_98 = l_Lean_Elab_getInfoTrees___at_Lean_Elab_Command_elabCommandTopLevel___spec__1___rarg(x_3, x_96); -x_99 = lean_ctor_get(x_98, 0); -lean_inc(x_99); -x_100 = lean_ctor_get(x_98, 1); -lean_inc(x_100); -lean_dec(x_98); -x_101 = lean_box(0); -x_102 = l_Lean_PersistentArray_forIn___at_Lean_Elab_Command_elabCommandTopLevel___spec__3(x_99, x_101, x_28, x_3, x_100); -lean_dec(x_99); -if (lean_obj_tag(x_102) == 0) +lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; +x_106 = lean_st_ref_get(x_3, x_105); +x_107 = lean_ctor_get(x_106, 0); +lean_inc(x_107); +x_108 = lean_ctor_get(x_106, 1); +lean_inc(x_108); +lean_dec(x_106); +x_109 = lean_ctor_get(x_107, 1); +lean_inc(x_109); +lean_dec(x_107); +x_110 = l_Lean_Elab_getInfoTrees___at_Lean_Elab_Command_elabCommandTopLevel___spec__1___rarg(x_3, x_108); +x_111 = lean_ctor_get(x_110, 0); +lean_inc(x_111); +x_112 = lean_ctor_get(x_110, 1); +lean_inc(x_112); +lean_dec(x_110); +x_113 = lean_box(0); +x_114 = l_Lean_PersistentArray_forIn___at_Lean_Elab_Command_elabCommandTopLevel___spec__3(x_111, x_113, x_28, x_3, x_112); +lean_dec(x_111); +if (lean_obj_tag(x_114) == 0) +{ +lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; uint8_t x_119; +x_115 = lean_ctor_get(x_114, 1); +lean_inc(x_115); +lean_dec(x_114); +x_116 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_4859____closed__5; +x_117 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Command_runLinters___spec__11(x_116, x_28, x_3, x_115); +x_118 = lean_ctor_get(x_117, 0); +lean_inc(x_118); +x_119 = lean_unbox(x_118); +lean_dec(x_118); +if (x_119 == 0) +{ +lean_object* x_120; lean_object* x_121; uint8_t x_122; +lean_dec(x_20); +x_120 = lean_ctor_get(x_117, 1); +lean_inc(x_120); +lean_dec(x_117); +x_121 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_30, x_109, x_35, x_113, x_28, x_3, x_120); +lean_dec(x_3); +x_122 = !lean_is_exclusive(x_121); +if (x_122 == 0) +{ +lean_object* x_123; +x_123 = lean_ctor_get(x_121, 0); +lean_dec(x_123); +lean_ctor_set_tag(x_121, 1); +lean_ctor_set(x_121, 0, x_104); +return x_121; +} +else +{ +lean_object* x_124; lean_object* x_125; +x_124 = lean_ctor_get(x_121, 1); +lean_inc(x_124); +lean_dec(x_121); +x_125 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_125, 0, x_104); +lean_ctor_set(x_125, 1, x_124); +return x_125; +} +} +else { if (lean_obj_tag(x_20) == 0) { -lean_object* x_103; lean_object* x_104; uint8_t x_105; -x_103 = lean_ctor_get(x_102, 1); -lean_inc(x_103); -lean_dec(x_102); -x_104 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_30, x_97, x_35, x_101, x_28, x_3, x_103); +lean_object* x_126; lean_object* x_127; uint8_t x_128; +x_126 = lean_ctor_get(x_117, 1); +lean_inc(x_126); +lean_dec(x_117); +x_127 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_30, x_109, x_35, x_113, x_28, x_3, x_126); lean_dec(x_3); -x_105 = !lean_is_exclusive(x_104); -if (x_105 == 0) +x_128 = !lean_is_exclusive(x_127); +if (x_128 == 0) { -lean_object* x_106; -x_106 = lean_ctor_get(x_104, 0); -lean_dec(x_106); -lean_ctor_set_tag(x_104, 1); -lean_ctor_set(x_104, 0, x_92); -return x_104; +lean_object* x_129; +x_129 = lean_ctor_get(x_127, 0); +lean_dec(x_129); +lean_ctor_set_tag(x_127, 1); +lean_ctor_set(x_127, 0, x_104); +return x_127; } else { -lean_object* x_107; lean_object* x_108; -x_107 = lean_ctor_get(x_104, 1); -lean_inc(x_107); -lean_dec(x_104); -x_108 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_108, 0, x_92); -lean_ctor_set(x_108, 1, x_107); -return x_108; +lean_object* x_130; lean_object* x_131; +x_130 = lean_ctor_get(x_127, 1); +lean_inc(x_130); +lean_dec(x_127); +x_131 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_131, 0, x_104); +lean_ctor_set(x_131, 1, x_130); +return x_131; } } else { -lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; uint8_t x_113; lean_object* x_114; lean_object* x_136; lean_object* x_137; -x_109 = lean_ctor_get(x_102, 1); -lean_inc(x_109); -lean_dec(x_102); -x_110 = lean_ctor_get(x_20, 0); -lean_inc(x_110); +lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; uint8_t x_136; lean_object* x_137; lean_object* x_160; lean_object* x_161; +x_132 = lean_ctor_get(x_117, 1); +lean_inc(x_132); +lean_dec(x_117); +x_133 = lean_ctor_get(x_20, 0); +lean_inc(x_133); lean_dec(x_20); -x_111 = lean_ctor_get(x_110, 1); -lean_inc(x_111); -lean_dec(x_110); -x_112 = lean_io_promise_result(x_111); -x_136 = lean_io_get_task_state(x_112, x_109); -x_137 = lean_ctor_get(x_136, 0); -lean_inc(x_137); -if (lean_obj_tag(x_137) == 2) +x_134 = lean_ctor_get(x_133, 1); +lean_inc(x_134); +lean_dec(x_133); +x_135 = lean_io_promise_result(x_134); +x_160 = lean_io_get_task_state(x_135, x_132); +x_161 = lean_ctor_get(x_160, 0); +lean_inc(x_161); +if (lean_obj_tag(x_161) == 2) { -lean_object* x_138; uint8_t x_139; -x_138 = lean_ctor_get(x_136, 1); -lean_inc(x_138); -lean_dec(x_136); -x_139 = 1; -x_113 = x_139; -x_114 = x_138; -goto block_135; +lean_object* x_162; uint8_t x_163; +x_162 = lean_ctor_get(x_160, 1); +lean_inc(x_162); +lean_dec(x_160); +x_163 = 1; +x_136 = x_163; +x_137 = x_162; +goto block_159; } else { -lean_object* x_140; uint8_t x_141; -lean_dec(x_137); -x_140 = lean_ctor_get(x_136, 1); -lean_inc(x_140); -lean_dec(x_136); -x_141 = 0; -x_113 = x_141; -x_114 = x_140; -goto block_135; +lean_object* x_164; uint8_t x_165; +lean_dec(x_161); +x_164 = lean_ctor_get(x_160, 1); +lean_inc(x_164); +lean_dec(x_160); +x_165 = 0; +x_136 = x_165; +x_137 = x_164; +goto block_159; } -block_135: +block_159: { -if (x_113 == 0) +if (x_136 == 0) { -lean_object* x_115; uint8_t x_116; -lean_dec(x_112); -x_115 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_30, x_97, x_35, x_101, x_28, x_3, x_114); +lean_object* x_138; uint8_t x_139; +lean_dec(x_135); +x_138 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_30, x_109, x_35, x_113, x_28, x_3, x_137); lean_dec(x_3); -x_116 = !lean_is_exclusive(x_115); -if (x_116 == 0) +x_139 = !lean_is_exclusive(x_138); +if (x_139 == 0) { -lean_object* x_117; -x_117 = lean_ctor_get(x_115, 0); -lean_dec(x_117); -lean_ctor_set_tag(x_115, 1); -lean_ctor_set(x_115, 0, x_92); -return x_115; +lean_object* x_140; +x_140 = lean_ctor_get(x_138, 0); +lean_dec(x_140); +lean_ctor_set_tag(x_138, 1); +lean_ctor_set(x_138, 0, x_104); +return x_138; } else { -lean_object* x_118; lean_object* x_119; -x_118 = lean_ctor_get(x_115, 1); -lean_inc(x_118); -lean_dec(x_115); -x_119 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_119, 0, x_92); -lean_ctor_set(x_119, 1, x_118); -return x_119; +lean_object* x_141; lean_object* x_142; +x_141 = lean_ctor_get(x_138, 1); +lean_inc(x_141); +lean_dec(x_138); +x_142 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_142, 0, x_104); +lean_ctor_set(x_142, 1, x_141); +return x_142; } } else { -lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; -x_120 = lean_task_get_own(x_112); -x_121 = lean_ctor_get(x_120, 1); -lean_inc(x_121); -lean_dec(x_120); -x_122 = lean_alloc_closure((void*)(l_Lean_Language_SnapshotTree_trace), 4, 1); -lean_closure_set(x_122, 0, x_121); -x_123 = l_Lean_Elab_Command_liftCoreM___rarg(x_122, x_28, x_3, x_114); -if (lean_obj_tag(x_123) == 0) +lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; +x_143 = lean_task_get_own(x_135); +x_144 = lean_ctor_get(x_143, 1); +lean_inc(x_144); +lean_dec(x_143); +x_145 = lean_thunk_get_own(x_144); +lean_dec(x_144); +x_146 = lean_alloc_closure((void*)(l_Lean_Language_SnapshotTree_trace), 4, 1); +lean_closure_set(x_146, 0, x_145); +x_147 = l_Lean_Elab_Command_liftCoreM___rarg(x_146, x_28, x_3, x_137); +if (lean_obj_tag(x_147) == 0) { -lean_object* x_124; lean_object* x_125; lean_object* x_126; uint8_t x_127; -x_124 = lean_ctor_get(x_123, 0); -lean_inc(x_124); -x_125 = lean_ctor_get(x_123, 1); -lean_inc(x_125); -lean_dec(x_123); -x_126 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_30, x_97, x_35, x_124, x_28, x_3, x_125); +lean_object* x_148; lean_object* x_149; lean_object* x_150; uint8_t x_151; +x_148 = lean_ctor_get(x_147, 0); +lean_inc(x_148); +x_149 = lean_ctor_get(x_147, 1); +lean_inc(x_149); +lean_dec(x_147); +x_150 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_30, x_109, x_35, x_148, x_28, x_3, x_149); lean_dec(x_3); -lean_dec(x_124); -x_127 = !lean_is_exclusive(x_126); -if (x_127 == 0) +lean_dec(x_148); +x_151 = !lean_is_exclusive(x_150); +if (x_151 == 0) { -lean_object* x_128; -x_128 = lean_ctor_get(x_126, 0); -lean_dec(x_128); -lean_ctor_set_tag(x_126, 1); -lean_ctor_set(x_126, 0, x_92); -return x_126; +lean_object* x_152; +x_152 = lean_ctor_get(x_150, 0); +lean_dec(x_152); +lean_ctor_set_tag(x_150, 1); +lean_ctor_set(x_150, 0, x_104); +return x_150; } else { -lean_object* x_129; lean_object* x_130; -x_129 = lean_ctor_get(x_126, 1); -lean_inc(x_129); -lean_dec(x_126); -x_130 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_130, 0, x_92); -lean_ctor_set(x_130, 1, x_129); -return x_130; +lean_object* x_153; lean_object* x_154; +x_153 = lean_ctor_get(x_150, 1); +lean_inc(x_153); +lean_dec(x_150); +x_154 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_154, 0, x_104); +lean_ctor_set(x_154, 1, x_153); +return x_154; } } else { -uint8_t x_131; -lean_dec(x_97); -lean_dec(x_92); +uint8_t x_155; +lean_dec(x_109); +lean_dec(x_104); lean_dec(x_35); lean_dec(x_30); lean_dec(x_28); lean_dec(x_3); -x_131 = !lean_is_exclusive(x_123); -if (x_131 == 0) +x_155 = !lean_is_exclusive(x_147); +if (x_155 == 0) { -return x_123; +return x_147; } else { -lean_object* x_132; lean_object* x_133; lean_object* x_134; -x_132 = lean_ctor_get(x_123, 0); -x_133 = lean_ctor_get(x_123, 1); -lean_inc(x_133); -lean_inc(x_132); -lean_dec(x_123); -x_134 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_134, 0, x_132); -lean_ctor_set(x_134, 1, x_133); -return x_134; +lean_object* x_156; lean_object* x_157; lean_object* x_158; +x_156 = lean_ctor_get(x_147, 0); +x_157 = lean_ctor_get(x_147, 1); +lean_inc(x_157); +lean_inc(x_156); +lean_dec(x_147); +x_158 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_158, 0, x_156); +lean_ctor_set(x_158, 1, x_157); +return x_158; +} } } } @@ -28451,330 +28468,373 @@ return x_134; } else { -uint8_t x_142; -lean_dec(x_97); -lean_dec(x_92); +uint8_t x_166; +lean_dec(x_109); +lean_dec(x_104); lean_dec(x_35); lean_dec(x_30); lean_dec(x_28); lean_dec(x_20); lean_dec(x_3); -x_142 = !lean_is_exclusive(x_102); -if (x_142 == 0) +x_166 = !lean_is_exclusive(x_114); +if (x_166 == 0) { -return x_102; +return x_114; } else { -lean_object* x_143; lean_object* x_144; lean_object* x_145; -x_143 = lean_ctor_get(x_102, 0); -x_144 = lean_ctor_get(x_102, 1); -lean_inc(x_144); -lean_inc(x_143); -lean_dec(x_102); -x_145 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_145, 0, x_143); -lean_ctor_set(x_145, 1, x_144); -return x_145; +lean_object* x_167; lean_object* x_168; lean_object* x_169; +x_167 = lean_ctor_get(x_114, 0); +x_168 = lean_ctor_get(x_114, 1); +lean_inc(x_168); +lean_inc(x_167); +lean_dec(x_114); +x_169 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_169, 0, x_167); +lean_ctor_set(x_169, 1, x_168); +return x_169; } } } } else { -lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_227; lean_object* x_228; lean_object* x_279; -x_160 = lean_ctor_get(x_26, 0); -x_161 = lean_ctor_get(x_26, 1); -x_162 = lean_ctor_get(x_26, 2); -x_163 = lean_ctor_get(x_26, 3); -x_164 = lean_ctor_get(x_26, 4); -x_165 = lean_ctor_get(x_26, 5); -x_166 = lean_ctor_get(x_26, 6); -x_167 = lean_ctor_get(x_26, 7); -lean_inc(x_167); -lean_inc(x_166); -lean_inc(x_165); -lean_inc(x_164); -lean_inc(x_163); -lean_inc(x_162); -lean_inc(x_161); -lean_inc(x_160); +lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_262; lean_object* x_263; lean_object* x_325; +x_184 = lean_ctor_get(x_26, 0); +x_185 = lean_ctor_get(x_26, 1); +x_186 = lean_ctor_get(x_26, 2); +x_187 = lean_ctor_get(x_26, 3); +x_188 = lean_ctor_get(x_26, 4); +x_189 = lean_ctor_get(x_26, 5); +x_190 = lean_ctor_get(x_26, 6); +x_191 = lean_ctor_get(x_26, 7); +lean_inc(x_191); +lean_inc(x_190); +lean_inc(x_189); +lean_inc(x_188); +lean_inc(x_187); +lean_inc(x_186); +lean_inc(x_185); +lean_inc(x_184); lean_dec(x_26); -x_168 = l___private_Lean_Elab_Command_0__Lean_Elab_Command_runCore___rarg___closed__4; -x_169 = lean_alloc_ctor(0, 8, 0); -lean_ctor_set(x_169, 0, x_160); -lean_ctor_set(x_169, 1, x_168); -lean_ctor_set(x_169, 2, x_162); -lean_ctor_set(x_169, 3, x_163); -lean_ctor_set(x_169, 4, x_164); -lean_ctor_set(x_169, 5, x_165); -lean_ctor_set(x_169, 6, x_166); -lean_ctor_set(x_169, 7, x_167); -x_170 = lean_st_ref_set(x_3, x_169, x_27); -x_171 = lean_ctor_get(x_170, 1); -lean_inc(x_171); -lean_dec(x_170); -x_172 = l_Lean_Elab_getResetInfoTrees___at___private_Lean_Elab_Command_0__Lean_Elab_Command_elabCommandUsing___spec__3___rarg(x_3, x_171); -x_173 = lean_ctor_get(x_172, 0); -lean_inc(x_173); -x_174 = lean_ctor_get(x_172, 1); -lean_inc(x_174); -lean_dec(x_172); +x_192 = l___private_Lean_Elab_Command_0__Lean_Elab_Command_runCore___rarg___closed__4; +x_193 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_193, 0, x_184); +lean_ctor_set(x_193, 1, x_192); +lean_ctor_set(x_193, 2, x_186); +lean_ctor_set(x_193, 3, x_187); +lean_ctor_set(x_193, 4, x_188); +lean_ctor_set(x_193, 5, x_189); +lean_ctor_set(x_193, 6, x_190); +lean_ctor_set(x_193, 7, x_191); +x_194 = lean_st_ref_set(x_3, x_193, x_27); +x_195 = lean_ctor_get(x_194, 1); +lean_inc(x_195); +lean_dec(x_194); +x_196 = l_Lean_Elab_getResetInfoTrees___at___private_Lean_Elab_Command_0__Lean_Elab_Command_elabCommandUsing___spec__3___rarg(x_3, x_195); +x_197 = lean_ctor_get(x_196, 0); +lean_inc(x_197); +x_198 = lean_ctor_get(x_196, 1); +lean_inc(x_198); +lean_dec(x_196); lean_inc(x_3); lean_inc(x_28); lean_inc(x_1); -x_279 = l_Lean_Elab_Command_elabCommand(x_1, x_28, x_3, x_174); -if (lean_obj_tag(x_279) == 0) -{ -lean_object* x_280; lean_object* x_281; lean_object* x_282; -x_280 = lean_ctor_get(x_279, 1); -lean_inc(x_280); -lean_dec(x_279); -x_281 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__3___closed__1; +x_325 = l_Lean_Elab_Command_elabCommand(x_1, x_28, x_3, x_198); +if (lean_obj_tag(x_325) == 0) +{ +lean_object* x_326; lean_object* x_327; lean_object* x_328; +x_326 = lean_ctor_get(x_325, 1); +lean_inc(x_326); +lean_dec(x_325); +x_327 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__3___closed__1; lean_inc(x_1); -x_282 = l_Lean_Syntax_findAux(x_281, x_1); -if (lean_obj_tag(x_282) == 0) +x_328 = l_Lean_Syntax_findAux(x_327, x_1); +if (lean_obj_tag(x_328) == 0) { -lean_object* x_283; lean_object* x_284; -x_283 = lean_alloc_closure((void*)(l_Lean_Elab_Command_runLinters), 4, 1); -lean_closure_set(x_283, 0, x_1); +lean_object* x_329; lean_object* x_330; +x_329 = lean_alloc_closure((void*)(l_Lean_Elab_Command_runLinters), 4, 1); +lean_closure_set(x_329, 0, x_1); lean_inc(x_3); lean_inc(x_28); -x_284 = l_Lean_Elab_withLogging___at_Lean_Elab_Command_elabCommand___spec__2(x_283, x_28, x_3, x_280); -if (lean_obj_tag(x_284) == 0) +x_330 = l_Lean_Elab_withLogging___at_Lean_Elab_Command_elabCommand___spec__2(x_329, x_28, x_3, x_326); +if (lean_obj_tag(x_330) == 0) { -lean_object* x_285; lean_object* x_286; -x_285 = lean_ctor_get(x_284, 0); -lean_inc(x_285); -x_286 = lean_ctor_get(x_284, 1); -lean_inc(x_286); -lean_dec(x_284); -x_175 = x_285; -x_176 = x_286; -goto block_226; +lean_object* x_331; lean_object* x_332; +x_331 = lean_ctor_get(x_330, 0); +lean_inc(x_331); +x_332 = lean_ctor_get(x_330, 1); +lean_inc(x_332); +lean_dec(x_330); +x_199 = x_331; +x_200 = x_332; +goto block_261; } else { -lean_object* x_287; lean_object* x_288; -x_287 = lean_ctor_get(x_284, 0); -lean_inc(x_287); -x_288 = lean_ctor_get(x_284, 1); -lean_inc(x_288); -lean_dec(x_284); -x_227 = x_287; -x_228 = x_288; -goto block_278; +lean_object* x_333; lean_object* x_334; +x_333 = lean_ctor_get(x_330, 0); +lean_inc(x_333); +x_334 = lean_ctor_get(x_330, 1); +lean_inc(x_334); +lean_dec(x_330); +x_262 = x_333; +x_263 = x_334; +goto block_324; } } else { -lean_object* x_289; -lean_dec(x_282); +lean_object* x_335; +lean_dec(x_328); lean_dec(x_1); -x_289 = lean_box(0); -x_175 = x_289; -x_176 = x_280; -goto block_226; +x_335 = lean_box(0); +x_199 = x_335; +x_200 = x_326; +goto block_261; } } else { -lean_object* x_290; lean_object* x_291; +lean_object* x_336; lean_object* x_337; lean_dec(x_1); -x_290 = lean_ctor_get(x_279, 0); -lean_inc(x_290); -x_291 = lean_ctor_get(x_279, 1); -lean_inc(x_291); -lean_dec(x_279); -x_227 = x_290; -x_228 = x_291; -goto block_278; -} -block_226: -{ -lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; -x_177 = lean_st_ref_get(x_3, x_176); -x_178 = lean_ctor_get(x_177, 0); -lean_inc(x_178); -x_179 = lean_ctor_get(x_177, 1); -lean_inc(x_179); -lean_dec(x_177); -x_180 = lean_ctor_get(x_178, 1); -lean_inc(x_180); -lean_dec(x_178); -x_181 = l_Lean_Elab_getInfoTrees___at_Lean_Elab_Command_elabCommandTopLevel___spec__1___rarg(x_3, x_179); -x_182 = lean_ctor_get(x_181, 0); -lean_inc(x_182); -x_183 = lean_ctor_get(x_181, 1); -lean_inc(x_183); -lean_dec(x_181); -x_184 = lean_box(0); -x_185 = l_Lean_PersistentArray_forIn___at_Lean_Elab_Command_elabCommandTopLevel___spec__3(x_182, x_184, x_28, x_3, x_183); -lean_dec(x_182); -if (lean_obj_tag(x_185) == 0) +x_336 = lean_ctor_get(x_325, 0); +lean_inc(x_336); +x_337 = lean_ctor_get(x_325, 1); +lean_inc(x_337); +lean_dec(x_325); +x_262 = x_336; +x_263 = x_337; +goto block_324; +} +block_261: +{ +lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; +x_201 = lean_st_ref_get(x_3, x_200); +x_202 = lean_ctor_get(x_201, 0); +lean_inc(x_202); +x_203 = lean_ctor_get(x_201, 1); +lean_inc(x_203); +lean_dec(x_201); +x_204 = lean_ctor_get(x_202, 1); +lean_inc(x_204); +lean_dec(x_202); +x_205 = l_Lean_Elab_getInfoTrees___at_Lean_Elab_Command_elabCommandTopLevel___spec__1___rarg(x_3, x_203); +x_206 = lean_ctor_get(x_205, 0); +lean_inc(x_206); +x_207 = lean_ctor_get(x_205, 1); +lean_inc(x_207); +lean_dec(x_205); +x_208 = lean_box(0); +x_209 = l_Lean_PersistentArray_forIn___at_Lean_Elab_Command_elabCommandTopLevel___spec__3(x_206, x_208, x_28, x_3, x_207); +lean_dec(x_206); +if (lean_obj_tag(x_209) == 0) { -if (lean_obj_tag(x_20) == 0) +lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; uint8_t x_214; +x_210 = lean_ctor_get(x_209, 1); +lean_inc(x_210); +lean_dec(x_209); +x_211 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_4859____closed__5; +x_212 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Command_runLinters___spec__11(x_211, x_28, x_3, x_210); +x_213 = lean_ctor_get(x_212, 0); +lean_inc(x_213); +x_214 = lean_unbox(x_213); +lean_dec(x_213); +if (x_214 == 0) { -lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; -x_186 = lean_ctor_get(x_185, 1); -lean_inc(x_186); -lean_dec(x_185); -x_187 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_161, x_180, x_173, x_184, x_28, x_3, x_186); +lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; +lean_dec(x_20); +x_215 = lean_ctor_get(x_212, 1); +lean_inc(x_215); +lean_dec(x_212); +x_216 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_185, x_204, x_197, x_208, x_28, x_3, x_215); lean_dec(x_3); -x_188 = lean_ctor_get(x_187, 1); -lean_inc(x_188); -if (lean_is_exclusive(x_187)) { - lean_ctor_release(x_187, 0); - lean_ctor_release(x_187, 1); - x_189 = x_187; +x_217 = lean_ctor_get(x_216, 1); +lean_inc(x_217); +if (lean_is_exclusive(x_216)) { + lean_ctor_release(x_216, 0); + lean_ctor_release(x_216, 1); + x_218 = x_216; } else { - lean_dec_ref(x_187); - x_189 = lean_box(0); + lean_dec_ref(x_216); + x_218 = lean_box(0); } -if (lean_is_scalar(x_189)) { - x_190 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_218)) { + x_219 = lean_alloc_ctor(0, 2, 0); } else { - x_190 = x_189; + x_219 = x_218; } -lean_ctor_set(x_190, 0, x_175); -lean_ctor_set(x_190, 1, x_188); -return x_190; +lean_ctor_set(x_219, 0, x_199); +lean_ctor_set(x_219, 1, x_217); +return x_219; } else { -lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; uint8_t x_195; lean_object* x_196; lean_object* x_216; lean_object* x_217; -x_191 = lean_ctor_get(x_185, 1); -lean_inc(x_191); -lean_dec(x_185); -x_192 = lean_ctor_get(x_20, 0); -lean_inc(x_192); -lean_dec(x_20); -x_193 = lean_ctor_get(x_192, 1); -lean_inc(x_193); -lean_dec(x_192); -x_194 = lean_io_promise_result(x_193); -x_216 = lean_io_get_task_state(x_194, x_191); -x_217 = lean_ctor_get(x_216, 0); -lean_inc(x_217); -if (lean_obj_tag(x_217) == 2) -{ -lean_object* x_218; uint8_t x_219; -x_218 = lean_ctor_get(x_216, 1); -lean_inc(x_218); -lean_dec(x_216); -x_219 = 1; -x_195 = x_219; -x_196 = x_218; -goto block_215; -} -else +if (lean_obj_tag(x_20) == 0) { -lean_object* x_220; uint8_t x_221; -lean_dec(x_217); -x_220 = lean_ctor_get(x_216, 1); +lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; +x_220 = lean_ctor_get(x_212, 1); lean_inc(x_220); -lean_dec(x_216); -x_221 = 0; -x_195 = x_221; -x_196 = x_220; -goto block_215; -} -block_215: -{ -if (x_195 == 0) -{ -lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; -lean_dec(x_194); -x_197 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_161, x_180, x_173, x_184, x_28, x_3, x_196); +lean_dec(x_212); +x_221 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_185, x_204, x_197, x_208, x_28, x_3, x_220); lean_dec(x_3); -x_198 = lean_ctor_get(x_197, 1); -lean_inc(x_198); -if (lean_is_exclusive(x_197)) { - lean_ctor_release(x_197, 0); - lean_ctor_release(x_197, 1); - x_199 = x_197; +x_222 = lean_ctor_get(x_221, 1); +lean_inc(x_222); +if (lean_is_exclusive(x_221)) { + lean_ctor_release(x_221, 0); + lean_ctor_release(x_221, 1); + x_223 = x_221; } else { - lean_dec_ref(x_197); - x_199 = lean_box(0); + lean_dec_ref(x_221); + x_223 = lean_box(0); } -if (lean_is_scalar(x_199)) { - x_200 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_223)) { + x_224 = lean_alloc_ctor(0, 2, 0); } else { - x_200 = x_199; + x_224 = x_223; } -lean_ctor_set(x_200, 0, x_175); -lean_ctor_set(x_200, 1, x_198); -return x_200; +lean_ctor_set(x_224, 0, x_199); +lean_ctor_set(x_224, 1, x_222); +return x_224; } else { -lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; -x_201 = lean_task_get_own(x_194); -x_202 = lean_ctor_get(x_201, 1); -lean_inc(x_202); -lean_dec(x_201); -x_203 = lean_alloc_closure((void*)(l_Lean_Language_SnapshotTree_trace), 4, 1); -lean_closure_set(x_203, 0, x_202); -x_204 = l_Lean_Elab_Command_liftCoreM___rarg(x_203, x_28, x_3, x_196); -if (lean_obj_tag(x_204) == 0) +lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; uint8_t x_229; lean_object* x_230; lean_object* x_251; lean_object* x_252; +x_225 = lean_ctor_get(x_212, 1); +lean_inc(x_225); +lean_dec(x_212); +x_226 = lean_ctor_get(x_20, 0); +lean_inc(x_226); +lean_dec(x_20); +x_227 = lean_ctor_get(x_226, 1); +lean_inc(x_227); +lean_dec(x_226); +x_228 = lean_io_promise_result(x_227); +x_251 = lean_io_get_task_state(x_228, x_225); +x_252 = lean_ctor_get(x_251, 0); +lean_inc(x_252); +if (lean_obj_tag(x_252) == 2) { -lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; -x_205 = lean_ctor_get(x_204, 0); -lean_inc(x_205); -x_206 = lean_ctor_get(x_204, 1); -lean_inc(x_206); -lean_dec(x_204); -x_207 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_161, x_180, x_173, x_205, x_28, x_3, x_206); +lean_object* x_253; uint8_t x_254; +x_253 = lean_ctor_get(x_251, 1); +lean_inc(x_253); +lean_dec(x_251); +x_254 = 1; +x_229 = x_254; +x_230 = x_253; +goto block_250; +} +else +{ +lean_object* x_255; uint8_t x_256; +lean_dec(x_252); +x_255 = lean_ctor_get(x_251, 1); +lean_inc(x_255); +lean_dec(x_251); +x_256 = 0; +x_229 = x_256; +x_230 = x_255; +goto block_250; +} +block_250: +{ +if (x_229 == 0) +{ +lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; +lean_dec(x_228); +x_231 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_185, x_204, x_197, x_208, x_28, x_3, x_230); lean_dec(x_3); -lean_dec(x_205); -x_208 = lean_ctor_get(x_207, 1); -lean_inc(x_208); -if (lean_is_exclusive(x_207)) { - lean_ctor_release(x_207, 0); - lean_ctor_release(x_207, 1); - x_209 = x_207; +x_232 = lean_ctor_get(x_231, 1); +lean_inc(x_232); +if (lean_is_exclusive(x_231)) { + lean_ctor_release(x_231, 0); + lean_ctor_release(x_231, 1); + x_233 = x_231; } else { - lean_dec_ref(x_207); - x_209 = lean_box(0); + lean_dec_ref(x_231); + x_233 = lean_box(0); } -if (lean_is_scalar(x_209)) { - x_210 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_233)) { + x_234 = lean_alloc_ctor(0, 2, 0); } else { - x_210 = x_209; + x_234 = x_233; } -lean_ctor_set(x_210, 0, x_175); -lean_ctor_set(x_210, 1, x_208); -return x_210; +lean_ctor_set(x_234, 0, x_199); +lean_ctor_set(x_234, 1, x_232); +return x_234; } else { -lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; -lean_dec(x_180); -lean_dec(x_175); -lean_dec(x_173); -lean_dec(x_161); +lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; +x_235 = lean_task_get_own(x_228); +x_236 = lean_ctor_get(x_235, 1); +lean_inc(x_236); +lean_dec(x_235); +x_237 = lean_thunk_get_own(x_236); +lean_dec(x_236); +x_238 = lean_alloc_closure((void*)(l_Lean_Language_SnapshotTree_trace), 4, 1); +lean_closure_set(x_238, 0, x_237); +x_239 = l_Lean_Elab_Command_liftCoreM___rarg(x_238, x_28, x_3, x_230); +if (lean_obj_tag(x_239) == 0) +{ +lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; +x_240 = lean_ctor_get(x_239, 0); +lean_inc(x_240); +x_241 = lean_ctor_get(x_239, 1); +lean_inc(x_241); +lean_dec(x_239); +x_242 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_185, x_204, x_197, x_240, x_28, x_3, x_241); +lean_dec(x_3); +lean_dec(x_240); +x_243 = lean_ctor_get(x_242, 1); +lean_inc(x_243); +if (lean_is_exclusive(x_242)) { + lean_ctor_release(x_242, 0); + lean_ctor_release(x_242, 1); + x_244 = x_242; +} else { + lean_dec_ref(x_242); + x_244 = lean_box(0); +} +if (lean_is_scalar(x_244)) { + x_245 = lean_alloc_ctor(0, 2, 0); +} else { + x_245 = x_244; +} +lean_ctor_set(x_245, 0, x_199); +lean_ctor_set(x_245, 1, x_243); +return x_245; +} +else +{ +lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; +lean_dec(x_204); +lean_dec(x_199); +lean_dec(x_197); +lean_dec(x_185); lean_dec(x_28); lean_dec(x_3); -x_211 = lean_ctor_get(x_204, 0); -lean_inc(x_211); -x_212 = lean_ctor_get(x_204, 1); -lean_inc(x_212); -if (lean_is_exclusive(x_204)) { - lean_ctor_release(x_204, 0); - lean_ctor_release(x_204, 1); - x_213 = x_204; +x_246 = lean_ctor_get(x_239, 0); +lean_inc(x_246); +x_247 = lean_ctor_get(x_239, 1); +lean_inc(x_247); +if (lean_is_exclusive(x_239)) { + lean_ctor_release(x_239, 0); + lean_ctor_release(x_239, 1); + x_248 = x_239; } else { - lean_dec_ref(x_204); - x_213 = lean_box(0); + lean_dec_ref(x_239); + x_248 = lean_box(0); } -if (lean_is_scalar(x_213)) { - x_214 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_248)) { + x_249 = lean_alloc_ctor(1, 2, 0); } else { - x_214 = x_213; + x_249 = x_248; +} +lean_ctor_set(x_249, 0, x_246); +lean_ctor_set(x_249, 1, x_247); +return x_249; } -lean_ctor_set(x_214, 0, x_211); -lean_ctor_set(x_214, 1, x_212); -return x_214; } } } @@ -28782,224 +28842,268 @@ return x_214; } else { -lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; -lean_dec(x_180); -lean_dec(x_175); -lean_dec(x_173); -lean_dec(x_161); +lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; +lean_dec(x_204); +lean_dec(x_199); +lean_dec(x_197); +lean_dec(x_185); lean_dec(x_28); lean_dec(x_20); lean_dec(x_3); -x_222 = lean_ctor_get(x_185, 0); -lean_inc(x_222); -x_223 = lean_ctor_get(x_185, 1); -lean_inc(x_223); -if (lean_is_exclusive(x_185)) { - lean_ctor_release(x_185, 0); - lean_ctor_release(x_185, 1); - x_224 = x_185; +x_257 = lean_ctor_get(x_209, 0); +lean_inc(x_257); +x_258 = lean_ctor_get(x_209, 1); +lean_inc(x_258); +if (lean_is_exclusive(x_209)) { + lean_ctor_release(x_209, 0); + lean_ctor_release(x_209, 1); + x_259 = x_209; } else { - lean_dec_ref(x_185); - x_224 = lean_box(0); + lean_dec_ref(x_209); + x_259 = lean_box(0); } -if (lean_is_scalar(x_224)) { - x_225 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_259)) { + x_260 = lean_alloc_ctor(1, 2, 0); } else { - x_225 = x_224; + x_260 = x_259; } -lean_ctor_set(x_225, 0, x_222); -lean_ctor_set(x_225, 1, x_223); -return x_225; +lean_ctor_set(x_260, 0, x_257); +lean_ctor_set(x_260, 1, x_258); +return x_260; } } -block_278: +block_324: { -lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; -x_229 = lean_st_ref_get(x_3, x_228); -x_230 = lean_ctor_get(x_229, 0); -lean_inc(x_230); -x_231 = lean_ctor_get(x_229, 1); -lean_inc(x_231); -lean_dec(x_229); -x_232 = lean_ctor_get(x_230, 1); -lean_inc(x_232); -lean_dec(x_230); -x_233 = l_Lean_Elab_getInfoTrees___at_Lean_Elab_Command_elabCommandTopLevel___spec__1___rarg(x_3, x_231); -x_234 = lean_ctor_get(x_233, 0); -lean_inc(x_234); -x_235 = lean_ctor_get(x_233, 1); -lean_inc(x_235); -lean_dec(x_233); -x_236 = lean_box(0); -x_237 = l_Lean_PersistentArray_forIn___at_Lean_Elab_Command_elabCommandTopLevel___spec__3(x_234, x_236, x_28, x_3, x_235); -lean_dec(x_234); -if (lean_obj_tag(x_237) == 0) +lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; +x_264 = lean_st_ref_get(x_3, x_263); +x_265 = lean_ctor_get(x_264, 0); +lean_inc(x_265); +x_266 = lean_ctor_get(x_264, 1); +lean_inc(x_266); +lean_dec(x_264); +x_267 = lean_ctor_get(x_265, 1); +lean_inc(x_267); +lean_dec(x_265); +x_268 = l_Lean_Elab_getInfoTrees___at_Lean_Elab_Command_elabCommandTopLevel___spec__1___rarg(x_3, x_266); +x_269 = lean_ctor_get(x_268, 0); +lean_inc(x_269); +x_270 = lean_ctor_get(x_268, 1); +lean_inc(x_270); +lean_dec(x_268); +x_271 = lean_box(0); +x_272 = l_Lean_PersistentArray_forIn___at_Lean_Elab_Command_elabCommandTopLevel___spec__3(x_269, x_271, x_28, x_3, x_270); +lean_dec(x_269); +if (lean_obj_tag(x_272) == 0) +{ +lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; uint8_t x_277; +x_273 = lean_ctor_get(x_272, 1); +lean_inc(x_273); +lean_dec(x_272); +x_274 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_4859____closed__5; +x_275 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Command_runLinters___spec__11(x_274, x_28, x_3, x_273); +x_276 = lean_ctor_get(x_275, 0); +lean_inc(x_276); +x_277 = lean_unbox(x_276); +lean_dec(x_276); +if (x_277 == 0) +{ +lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; +lean_dec(x_20); +x_278 = lean_ctor_get(x_275, 1); +lean_inc(x_278); +lean_dec(x_275); +x_279 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_185, x_267, x_197, x_271, x_28, x_3, x_278); +lean_dec(x_3); +x_280 = lean_ctor_get(x_279, 1); +lean_inc(x_280); +if (lean_is_exclusive(x_279)) { + lean_ctor_release(x_279, 0); + lean_ctor_release(x_279, 1); + x_281 = x_279; +} else { + lean_dec_ref(x_279); + x_281 = lean_box(0); +} +if (lean_is_scalar(x_281)) { + x_282 = lean_alloc_ctor(1, 2, 0); +} else { + x_282 = x_281; + lean_ctor_set_tag(x_282, 1); +} +lean_ctor_set(x_282, 0, x_262); +lean_ctor_set(x_282, 1, x_280); +return x_282; +} +else { if (lean_obj_tag(x_20) == 0) { -lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; -x_238 = lean_ctor_get(x_237, 1); -lean_inc(x_238); -lean_dec(x_237); -x_239 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_161, x_232, x_173, x_236, x_28, x_3, x_238); +lean_object* x_283; lean_object* x_284; lean_object* x_285; lean_object* x_286; lean_object* x_287; +x_283 = lean_ctor_get(x_275, 1); +lean_inc(x_283); +lean_dec(x_275); +x_284 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_185, x_267, x_197, x_271, x_28, x_3, x_283); lean_dec(x_3); -x_240 = lean_ctor_get(x_239, 1); -lean_inc(x_240); -if (lean_is_exclusive(x_239)) { - lean_ctor_release(x_239, 0); - lean_ctor_release(x_239, 1); - x_241 = x_239; +x_285 = lean_ctor_get(x_284, 1); +lean_inc(x_285); +if (lean_is_exclusive(x_284)) { + lean_ctor_release(x_284, 0); + lean_ctor_release(x_284, 1); + x_286 = x_284; } else { - lean_dec_ref(x_239); - x_241 = lean_box(0); + lean_dec_ref(x_284); + x_286 = lean_box(0); } -if (lean_is_scalar(x_241)) { - x_242 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_286)) { + x_287 = lean_alloc_ctor(1, 2, 0); } else { - x_242 = x_241; - lean_ctor_set_tag(x_242, 1); + x_287 = x_286; + lean_ctor_set_tag(x_287, 1); } -lean_ctor_set(x_242, 0, x_227); -lean_ctor_set(x_242, 1, x_240); -return x_242; +lean_ctor_set(x_287, 0, x_262); +lean_ctor_set(x_287, 1, x_285); +return x_287; } else { -lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; uint8_t x_247; lean_object* x_248; lean_object* x_268; lean_object* x_269; -x_243 = lean_ctor_get(x_237, 1); -lean_inc(x_243); -lean_dec(x_237); -x_244 = lean_ctor_get(x_20, 0); -lean_inc(x_244); +lean_object* x_288; lean_object* x_289; lean_object* x_290; lean_object* x_291; uint8_t x_292; lean_object* x_293; lean_object* x_314; lean_object* x_315; +x_288 = lean_ctor_get(x_275, 1); +lean_inc(x_288); +lean_dec(x_275); +x_289 = lean_ctor_get(x_20, 0); +lean_inc(x_289); lean_dec(x_20); -x_245 = lean_ctor_get(x_244, 1); -lean_inc(x_245); -lean_dec(x_244); -x_246 = lean_io_promise_result(x_245); -x_268 = lean_io_get_task_state(x_246, x_243); -x_269 = lean_ctor_get(x_268, 0); -lean_inc(x_269); -if (lean_obj_tag(x_269) == 2) -{ -lean_object* x_270; uint8_t x_271; -x_270 = lean_ctor_get(x_268, 1); -lean_inc(x_270); -lean_dec(x_268); -x_271 = 1; -x_247 = x_271; -x_248 = x_270; -goto block_267; +x_290 = lean_ctor_get(x_289, 1); +lean_inc(x_290); +lean_dec(x_289); +x_291 = lean_io_promise_result(x_290); +x_314 = lean_io_get_task_state(x_291, x_288); +x_315 = lean_ctor_get(x_314, 0); +lean_inc(x_315); +if (lean_obj_tag(x_315) == 2) +{ +lean_object* x_316; uint8_t x_317; +x_316 = lean_ctor_get(x_314, 1); +lean_inc(x_316); +lean_dec(x_314); +x_317 = 1; +x_292 = x_317; +x_293 = x_316; +goto block_313; } else { -lean_object* x_272; uint8_t x_273; -lean_dec(x_269); -x_272 = lean_ctor_get(x_268, 1); -lean_inc(x_272); -lean_dec(x_268); -x_273 = 0; -x_247 = x_273; -x_248 = x_272; -goto block_267; +lean_object* x_318; uint8_t x_319; +lean_dec(x_315); +x_318 = lean_ctor_get(x_314, 1); +lean_inc(x_318); +lean_dec(x_314); +x_319 = 0; +x_292 = x_319; +x_293 = x_318; +goto block_313; } -block_267: +block_313: { -if (x_247 == 0) +if (x_292 == 0) { -lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; -lean_dec(x_246); -x_249 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_161, x_232, x_173, x_236, x_28, x_3, x_248); +lean_object* x_294; lean_object* x_295; lean_object* x_296; lean_object* x_297; +lean_dec(x_291); +x_294 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_185, x_267, x_197, x_271, x_28, x_3, x_293); lean_dec(x_3); -x_250 = lean_ctor_get(x_249, 1); -lean_inc(x_250); -if (lean_is_exclusive(x_249)) { - lean_ctor_release(x_249, 0); - lean_ctor_release(x_249, 1); - x_251 = x_249; +x_295 = lean_ctor_get(x_294, 1); +lean_inc(x_295); +if (lean_is_exclusive(x_294)) { + lean_ctor_release(x_294, 0); + lean_ctor_release(x_294, 1); + x_296 = x_294; } else { - lean_dec_ref(x_249); - x_251 = lean_box(0); + lean_dec_ref(x_294); + x_296 = lean_box(0); } -if (lean_is_scalar(x_251)) { - x_252 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_296)) { + x_297 = lean_alloc_ctor(1, 2, 0); } else { - x_252 = x_251; - lean_ctor_set_tag(x_252, 1); + x_297 = x_296; + lean_ctor_set_tag(x_297, 1); } -lean_ctor_set(x_252, 0, x_227); -lean_ctor_set(x_252, 1, x_250); -return x_252; +lean_ctor_set(x_297, 0, x_262); +lean_ctor_set(x_297, 1, x_295); +return x_297; } else { -lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; -x_253 = lean_task_get_own(x_246); -x_254 = lean_ctor_get(x_253, 1); -lean_inc(x_254); -lean_dec(x_253); -x_255 = lean_alloc_closure((void*)(l_Lean_Language_SnapshotTree_trace), 4, 1); -lean_closure_set(x_255, 0, x_254); -x_256 = l_Lean_Elab_Command_liftCoreM___rarg(x_255, x_28, x_3, x_248); -if (lean_obj_tag(x_256) == 0) -{ -lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; -x_257 = lean_ctor_get(x_256, 0); -lean_inc(x_257); -x_258 = lean_ctor_get(x_256, 1); -lean_inc(x_258); -lean_dec(x_256); -x_259 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_161, x_232, x_173, x_257, x_28, x_3, x_258); +lean_object* x_298; lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; +x_298 = lean_task_get_own(x_291); +x_299 = lean_ctor_get(x_298, 1); +lean_inc(x_299); +lean_dec(x_298); +x_300 = lean_thunk_get_own(x_299); +lean_dec(x_299); +x_301 = lean_alloc_closure((void*)(l_Lean_Language_SnapshotTree_trace), 4, 1); +lean_closure_set(x_301, 0, x_300); +x_302 = l_Lean_Elab_Command_liftCoreM___rarg(x_301, x_28, x_3, x_293); +if (lean_obj_tag(x_302) == 0) +{ +lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; lean_object* x_307; lean_object* x_308; +x_303 = lean_ctor_get(x_302, 0); +lean_inc(x_303); +x_304 = lean_ctor_get(x_302, 1); +lean_inc(x_304); +lean_dec(x_302); +x_305 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_185, x_267, x_197, x_303, x_28, x_3, x_304); lean_dec(x_3); -lean_dec(x_257); -x_260 = lean_ctor_get(x_259, 1); -lean_inc(x_260); -if (lean_is_exclusive(x_259)) { - lean_ctor_release(x_259, 0); - lean_ctor_release(x_259, 1); - x_261 = x_259; +lean_dec(x_303); +x_306 = lean_ctor_get(x_305, 1); +lean_inc(x_306); +if (lean_is_exclusive(x_305)) { + lean_ctor_release(x_305, 0); + lean_ctor_release(x_305, 1); + x_307 = x_305; } else { - lean_dec_ref(x_259); - x_261 = lean_box(0); + lean_dec_ref(x_305); + x_307 = lean_box(0); } -if (lean_is_scalar(x_261)) { - x_262 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_307)) { + x_308 = lean_alloc_ctor(1, 2, 0); } else { - x_262 = x_261; - lean_ctor_set_tag(x_262, 1); + x_308 = x_307; + lean_ctor_set_tag(x_308, 1); } -lean_ctor_set(x_262, 0, x_227); -lean_ctor_set(x_262, 1, x_260); -return x_262; +lean_ctor_set(x_308, 0, x_262); +lean_ctor_set(x_308, 1, x_306); +return x_308; } else { -lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; -lean_dec(x_232); -lean_dec(x_227); -lean_dec(x_173); -lean_dec(x_161); +lean_object* x_309; lean_object* x_310; lean_object* x_311; lean_object* x_312; +lean_dec(x_267); +lean_dec(x_262); +lean_dec(x_197); +lean_dec(x_185); lean_dec(x_28); lean_dec(x_3); -x_263 = lean_ctor_get(x_256, 0); -lean_inc(x_263); -x_264 = lean_ctor_get(x_256, 1); -lean_inc(x_264); -if (lean_is_exclusive(x_256)) { - lean_ctor_release(x_256, 0); - lean_ctor_release(x_256, 1); - x_265 = x_256; +x_309 = lean_ctor_get(x_302, 0); +lean_inc(x_309); +x_310 = lean_ctor_get(x_302, 1); +lean_inc(x_310); +if (lean_is_exclusive(x_302)) { + lean_ctor_release(x_302, 0); + lean_ctor_release(x_302, 1); + x_311 = x_302; } else { - lean_dec_ref(x_256); - x_265 = lean_box(0); + lean_dec_ref(x_302); + x_311 = lean_box(0); } -if (lean_is_scalar(x_265)) { - x_266 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_311)) { + x_312 = lean_alloc_ctor(1, 2, 0); } else { - x_266 = x_265; + x_312 = x_311; +} +lean_ctor_set(x_312, 0, x_309); +lean_ctor_set(x_312, 1, x_310); +return x_312; } -lean_ctor_set(x_266, 0, x_263); -lean_ctor_set(x_266, 1, x_264); -return x_266; } } } @@ -29007,34 +29111,34 @@ return x_266; } else { -lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; -lean_dec(x_232); -lean_dec(x_227); -lean_dec(x_173); -lean_dec(x_161); +lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; +lean_dec(x_267); +lean_dec(x_262); +lean_dec(x_197); +lean_dec(x_185); lean_dec(x_28); lean_dec(x_20); lean_dec(x_3); -x_274 = lean_ctor_get(x_237, 0); -lean_inc(x_274); -x_275 = lean_ctor_get(x_237, 1); -lean_inc(x_275); -if (lean_is_exclusive(x_237)) { - lean_ctor_release(x_237, 0); - lean_ctor_release(x_237, 1); - x_276 = x_237; +x_320 = lean_ctor_get(x_272, 0); +lean_inc(x_320); +x_321 = lean_ctor_get(x_272, 1); +lean_inc(x_321); +if (lean_is_exclusive(x_272)) { + lean_ctor_release(x_272, 0); + lean_ctor_release(x_272, 1); + x_322 = x_272; } else { - lean_dec_ref(x_237); - x_276 = lean_box(0); + lean_dec_ref(x_272); + x_322 = lean_box(0); } -if (lean_is_scalar(x_276)) { - x_277 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_322)) { + x_323 = lean_alloc_ctor(1, 2, 0); } else { - x_277 = x_276; + x_323 = x_322; } -lean_ctor_set(x_277, 0, x_274); -lean_ctor_set(x_277, 1, x_275); -return x_277; +lean_ctor_set(x_323, 0, x_320); +lean_ctor_set(x_323, 1, x_321); +return x_323; } } } @@ -33648,7 +33752,7 @@ static lean_object* _init_l_Lean_Elab_Command_modifyScope___closed__4() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Elab_Command_modifyScope___closed__1; x_2 = l_Lean_Elab_Command_modifyScope___closed__2; -x_3 = lean_unsigned_to_nat(689u); +x_3 = lean_unsigned_to_nat(690u); x_4 = lean_unsigned_to_nat(16u); x_5 = l_Lean_Elab_Command_modifyScope___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -35098,5412 +35202,1870 @@ lean_dec(x_1); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(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___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___spec__1(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { _start: { -lean_object* x_5; 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_5 = l_Lean_Elab_Command_getRef(x_2, x_3, x_4); -x_6 = lean_ctor_get(x_5, 0); -lean_inc(x_6); -x_7 = lean_ctor_get(x_5, 1); -lean_inc(x_7); -lean_dec(x_5); -x_8 = lean_ctor_get(x_2, 4); -lean_inc(x_8); -lean_inc(x_8); -x_9 = l_Lean_Elab_getBetterRef(x_6, x_8); -lean_dec(x_6); -x_10 = l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1(x_1, x_2, x_3, x_7); -x_11 = !lean_is_exclusive(x_10); -if (x_11 == 0) -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; -x_12 = lean_ctor_get(x_10, 0); -x_13 = lean_ctor_get(x_10, 1); -x_14 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_12, x_8, x_2, x_3, x_13); -lean_dec(x_2); -x_15 = !lean_is_exclusive(x_14); -if (x_15 == 0) +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) { -lean_object* x_16; -x_16 = lean_ctor_get(x_14, 0); -lean_ctor_set(x_10, 1, x_16); -lean_ctor_set(x_10, 0, x_9); -lean_ctor_set_tag(x_14, 1); -lean_ctor_set(x_14, 0, x_10); -return x_14; +lean_inc(x_5); +return x_5; } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_14, 0); -x_18 = lean_ctor_get(x_14, 1); -lean_inc(x_18); -lean_inc(x_17); -lean_dec(x_14); -lean_ctor_set(x_10, 1, x_17); -lean_ctor_set(x_10, 0, x_9); -x_19 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_19, 0, x_10); -lean_ctor_set(x_19, 1, x_18); -return x_19; -} +lean_object* x_7; uint8_t x_8; lean_object* x_9; +x_7 = lean_array_uget(x_2, x_4); +x_8 = lean_ctor_get_uint8(x_7, sizeof(void*)*5 + 1); +x_9 = lean_box(x_8); +if (lean_obj_tag(x_9) == 2) +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_10 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_10, 0, x_7); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = lean_box(0); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_11); +lean_ctor_set(x_13, 1, x_12); +return x_13; } else { -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_20 = lean_ctor_get(x_10, 0); -x_21 = lean_ctor_get(x_10, 1); -lean_inc(x_21); -lean_inc(x_20); -lean_dec(x_10); -x_22 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_20, x_8, x_2, x_3, x_21); -lean_dec(x_2); -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -x_24 = lean_ctor_get(x_22, 1); -lean_inc(x_24); -if (lean_is_exclusive(x_22)) { - lean_ctor_release(x_22, 0); - lean_ctor_release(x_22, 1); - x_25 = x_22; -} else { - lean_dec_ref(x_22); - x_25 = lean_box(0); +size_t x_14; size_t x_15; +lean_dec(x_9); +lean_dec(x_7); +x_14 = 1; +x_15 = lean_usize_add(x_4, x_14); +{ +size_t _tmp_3 = x_15; +lean_object* _tmp_4 = x_1; +x_4 = _tmp_3; +x_5 = _tmp_4; } -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_9); -lean_ctor_set(x_26, 1, x_23); -if (lean_is_scalar(x_25)) { - x_27 = lean_alloc_ctor(1, 2, 0); -} else { - x_27 = x_25; - lean_ctor_set_tag(x_27, 1); +goto _start; } -lean_ctor_set(x_27, 0, x_26); -lean_ctor_set(x_27, 1, x_24); -return x_27; } } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__1() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___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_1; -x_1 = lean_mk_string_unchecked("invalid declaration name '", 26, 26); -return x_1; -} +lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_8 = lean_st_ref_take(x_6, x_7); +x_9 = lean_ctor_get(x_8, 0); +lean_inc(x_9); +x_10 = lean_ctor_get(x_8, 1); +lean_inc(x_10); +lean_dec(x_8); +x_11 = !lean_is_exclusive(x_9); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_12 = lean_ctor_get(x_9, 5); +x_13 = lean_ctor_get(x_9, 6); +x_14 = l_Lean_MessageLog_append(x_12, x_1); +x_15 = !lean_is_exclusive(x_13); +if (x_15 == 0) +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; +x_16 = lean_ctor_get(x_13, 1); +x_17 = lean_ctor_get(x_2, 1); +x_18 = l_Lean_PersistentArray_append___rarg(x_16, x_17); +lean_ctor_set(x_13, 1, x_18); +lean_ctor_set(x_9, 5, x_14); +x_19 = lean_st_ref_set(x_6, x_9, x_10); +x_20 = !lean_is_exclusive(x_19); +if (x_20 == 0) +{ +lean_object* x_21; +x_21 = lean_ctor_get(x_19, 0); +lean_dec(x_21); +lean_ctor_set(x_19, 0, x_3); +return x_19; } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__2() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +lean_object* x_22; lean_object* x_23; +x_22 = lean_ctor_get(x_19, 1); +lean_inc(x_22); +lean_dec(x_19); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_3); +lean_ctor_set(x_23, 1, x_22); +return x_23; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__3() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("', structure '", 14, 14); -return x_1; +uint8_t x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_24 = lean_ctor_get_uint8(x_13, sizeof(void*)*2); +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_ctor_get(x_2, 1); +x_28 = l_Lean_PersistentArray_append___rarg(x_26, x_27); +x_29 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_29, 0, x_25); +lean_ctor_set(x_29, 1, x_28); +lean_ctor_set_uint8(x_29, sizeof(void*)*2, x_24); +lean_ctor_set(x_9, 6, x_29); +lean_ctor_set(x_9, 5, x_14); +x_30 = lean_st_ref_set(x_6, x_9, x_10); +x_31 = lean_ctor_get(x_30, 1); +lean_inc(x_31); +if (lean_is_exclusive(x_30)) { + lean_ctor_release(x_30, 0); + lean_ctor_release(x_30, 1); + x_32 = x_30; +} else { + lean_dec_ref(x_30); + x_32 = lean_box(0); } +if (lean_is_scalar(x_32)) { + x_33 = lean_alloc_ctor(0, 2, 0); +} else { + x_33 = x_32; } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__3; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +lean_ctor_set(x_33, 0, x_3); +lean_ctor_set(x_33, 1, x_31); +return x_33; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__5() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("' has field '", 13, 13); -return x_1; +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_34 = lean_ctor_get(x_9, 0); +x_35 = lean_ctor_get(x_9, 1); +x_36 = lean_ctor_get(x_9, 2); +x_37 = lean_ctor_get(x_9, 3); +x_38 = lean_ctor_get(x_9, 4); +x_39 = lean_ctor_get(x_9, 5); +x_40 = lean_ctor_get(x_9, 6); +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_dec(x_9); +x_41 = l_Lean_MessageLog_append(x_39, x_1); +x_42 = lean_ctor_get_uint8(x_40, sizeof(void*)*2); +x_43 = lean_ctor_get(x_40, 0); +lean_inc(x_43); +x_44 = lean_ctor_get(x_40, 1); +lean_inc(x_44); +if (lean_is_exclusive(x_40)) { + lean_ctor_release(x_40, 0); + lean_ctor_release(x_40, 1); + x_45 = x_40; +} else { + lean_dec_ref(x_40); + x_45 = lean_box(0); } +x_46 = lean_ctor_get(x_2, 1); +x_47 = l_Lean_PersistentArray_append___rarg(x_44, x_46); +if (lean_is_scalar(x_45)) { + x_48 = lean_alloc_ctor(0, 2, 1); +} else { + x_48 = x_45; } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__5; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +lean_ctor_set(x_48, 0, x_43); +lean_ctor_set(x_48, 1, x_47); +lean_ctor_set_uint8(x_48, sizeof(void*)*2, x_42); +x_49 = lean_alloc_ctor(0, 7, 0); +lean_ctor_set(x_49, 0, x_34); +lean_ctor_set(x_49, 1, x_35); +lean_ctor_set(x_49, 2, x_36); +lean_ctor_set(x_49, 3, x_37); +lean_ctor_set(x_49, 4, x_38); +lean_ctor_set(x_49, 5, x_41); +lean_ctor_set(x_49, 6, x_48); +x_50 = lean_st_ref_set(x_6, x_49, x_10); +x_51 = lean_ctor_get(x_50, 1); +lean_inc(x_51); +if (lean_is_exclusive(x_50)) { + lean_ctor_release(x_50, 0); + lean_ctor_release(x_50, 1); + x_52 = x_50; +} else { + lean_dec_ref(x_50); + x_52 = lean_box(0); } +if (lean_is_scalar(x_52)) { + x_53 = lean_alloc_ctor(0, 2, 0); +} else { + x_53 = x_52; } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__7() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("'", 1, 1); -return x_1; +lean_ctor_set(x_53, 0, x_3); +lean_ctor_set(x_53, 1, x_51); +return x_53; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__8() { +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___lambda__2(lean_object* x_1) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__7; -x_2 = l_Lean_stringToMessageData(x_1); +lean_object* x_2; +x_2 = lean_box(0); return x_2; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5(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) { +static lean_object* _init_l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___closed__1() { _start: { -uint8_t x_10; -x_10 = lean_usize_dec_lt(x_5, x_4); -if (x_10 == 0) -{ -lean_object* x_11; -lean_dec(x_7); -lean_dec(x_2); -lean_dec(x_1); -x_11 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_11, 0, x_6); -lean_ctor_set(x_11, 1, x_9); -return x_11; -} -else -{ -lean_object* x_12; lean_object* x_13; uint8_t x_14; -lean_dec(x_6); -x_12 = lean_array_uget(x_3, x_5); -lean_inc(x_12); -lean_inc(x_2); -x_13 = l_Lean_Name_append(x_2, x_12); -x_14 = lean_name_eq(x_13, x_1); -lean_dec(x_13); -if (x_14 == 0) -{ -size_t x_15; size_t x_16; lean_object* x_17; -lean_dec(x_12); -x_15 = 1; -x_16 = lean_usize_add(x_5, x_15); -x_17 = lean_box(0); -x_5 = x_16; -x_6 = x_17; -goto _start; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = lean_box(0); +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; } -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; uint8_t x_33; -x_19 = l_Lean_MessageData_ofName(x_1); -x_20 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__2; -x_21 = lean_alloc_ctor(7, 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_Elab_Command_expandDeclId___spec__5___closed__4; -x_23 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_23, 0, x_21); -lean_ctor_set(x_23, 1, x_22); -x_24 = l_Lean_MessageData_ofName(x_2); -x_25 = lean_alloc_ctor(7, 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_Lean_Elab_Command_expandDeclId___spec__5___closed__6; -x_27 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_26); -x_28 = l_Lean_MessageData_ofName(x_12); -x_29 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_29, 0, x_27); -lean_ctor_set(x_29, 1, x_28); -x_30 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__8; -x_31 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_31, 0, x_29); -lean_ctor_set(x_31, 1, x_30); -x_32 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_31, x_7, x_8, x_9); -x_33 = !lean_is_exclusive(x_32); -if (x_33 == 0) -{ -return x_32; } -else +static lean_object* _init_l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___closed__2() { +_start: { -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_32, 0); -x_35 = lean_ctor_get(x_32, 1); -lean_inc(x_35); -lean_inc(x_34); -lean_dec(x_32); -x_36 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_36, 0, x_34); -lean_ctor_set(x_36, 1, x_35); -return x_36; -} +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___lambda__2___boxed), 1, 0); +return x_1; } } +static lean_object* _init_l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___closed__2; +x_2 = lean_box(0); +x_3 = lean_apply_1(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_checkIfShadowingStructureField___at_Lean_Elab_Command_expandDeclId___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_Elab_Command_0__Lean_liftCommandElabMCore___rarg(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -if (lean_obj_tag(x_1) == 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); -x_6 = lean_st_ref_get(x_3, x_4); +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; lean_object* x_10; uint8_t x_11; +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; lean_object* x_31; uint8_t x_32; x_8 = lean_ctor_get(x_6, 0); x_9 = lean_ctor_get(x_6, 1); -x_10 = lean_ctor_get(x_8, 0); +x_10 = lean_ctor_get(x_3, 0); +x_11 = lean_ctor_get(x_3, 1); +x_12 = lean_ctor_get(x_3, 2); +x_13 = lean_ctor_get(x_3, 3); +x_14 = lean_ctor_get(x_3, 4); +x_15 = lean_ctor_get(x_3, 5); +x_16 = lean_ctor_get(x_3, 10); +x_17 = lean_ctor_get(x_3, 11); +x_18 = lean_ctor_get_uint8(x_3, sizeof(void*)*12 + 1); +x_19 = lean_box(0); +x_20 = lean_box(0); +x_21 = lean_unsigned_to_nat(0u); +lean_inc(x_17); +lean_inc(x_15); +lean_inc(x_16); +lean_inc(x_13); +lean_inc(x_11); lean_inc(x_10); +x_22 = lean_alloc_ctor(0, 10, 1); +lean_ctor_set(x_22, 0, x_10); +lean_ctor_set(x_22, 1, x_11); +lean_ctor_set(x_22, 2, x_13); +lean_ctor_set(x_22, 3, x_21); +lean_ctor_set(x_22, 4, x_19); +lean_ctor_set(x_22, 5, x_16); +lean_ctor_set(x_22, 6, x_15); +lean_ctor_set(x_22, 7, x_20); +lean_ctor_set(x_22, 8, x_20); +lean_ctor_set(x_22, 9, x_17); +lean_ctor_set_uint8(x_22, sizeof(void*)*10, x_18); +x_23 = lean_ctor_get(x_8, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_8, 1); +lean_inc(x_24); +x_25 = lean_ctor_get(x_8, 2); +lean_inc(x_25); +x_26 = lean_ctor_get(x_8, 6); +lean_inc(x_26); lean_dec(x_8); -lean_inc(x_5); -x_11 = l_Lean_isStructure(x_10, x_5); -lean_dec(x_10); -if (x_11 == 0) -{ -lean_object* x_12; -lean_dec(x_5); -lean_dec(x_2); -lean_dec(x_1); -x_12 = lean_box(0); -lean_ctor_set(x_6, 0, x_12); -return x_6; -} -else +x_27 = l_Lean_Elab_Command_instInhabitedScope___closed__2; +x_28 = lean_box(0); +x_29 = l_Lean_Elab_Command_mkState___closed__1; +x_30 = 0; +lean_inc(x_12); +x_31 = lean_alloc_ctor(0, 9, 1); +lean_ctor_set(x_31, 0, x_27); +lean_ctor_set(x_31, 1, x_12); +lean_ctor_set(x_31, 2, x_28); +lean_ctor_set(x_31, 3, x_19); +lean_ctor_set(x_31, 4, x_19); +lean_ctor_set(x_31, 5, x_29); +lean_ctor_set(x_31, 6, x_29); +lean_ctor_set(x_31, 7, x_19); +lean_ctor_set(x_31, 8, x_19); +lean_ctor_set_uint8(x_31, sizeof(void*)*9, x_30); +lean_ctor_set_tag(x_6, 1); +lean_ctor_set(x_6, 1, x_19); +lean_ctor_set(x_6, 0, x_31); +x_32 = !lean_is_exclusive(x_26); +if (x_32 == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; size_t x_19; size_t x_20; lean_object* x_21; lean_object* x_22; -lean_free_object(x_6); -x_13 = lean_st_ref_get(x_3, x_9); -x_14 = lean_ctor_get(x_13, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_13, 1); -lean_inc(x_15); -lean_dec(x_13); -x_16 = lean_ctor_get(x_14, 0); -lean_inc(x_16); -lean_dec(x_14); -x_17 = 1; -lean_inc(x_5); -x_18 = l_Lean_getStructureFieldsFlattened(x_16, x_5, x_17); -lean_dec(x_16); -x_19 = lean_array_size(x_18); -x_20 = 0; -x_21 = lean_box(0); -x_22 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5(x_1, x_5, x_18, x_19, x_20, x_21, x_2, x_3, x_15); -lean_dec(x_18); -if (lean_obj_tag(x_22) == 0) -{ -uint8_t x_23; -x_23 = !lean_is_exclusive(x_22); -if (x_23 == 0) -{ -lean_object* x_24; -x_24 = lean_ctor_get(x_22, 0); -lean_dec(x_24); -lean_ctor_set(x_22, 0, x_21); -return x_22; -} -else -{ -lean_object* x_25; lean_object* x_26; -x_25 = lean_ctor_get(x_22, 1); -lean_inc(x_25); -lean_dec(x_22); -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_21); -lean_ctor_set(x_26, 1, x_25); -return x_26; -} -} -else -{ -uint8_t x_27; -x_27 = !lean_is_exclusive(x_22); -if (x_27 == 0) -{ -return x_22; -} -else -{ -lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_28 = lean_ctor_get(x_22, 0); -x_29 = lean_ctor_get(x_22, 1); -lean_inc(x_29); -lean_inc(x_28); -lean_dec(x_22); -x_30 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_30, 0, x_28); -lean_ctor_set(x_30, 1, x_29); -return x_30; -} -} -} -} -else -{ -lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; -x_31 = lean_ctor_get(x_6, 0); -x_32 = lean_ctor_get(x_6, 1); -lean_inc(x_32); -lean_inc(x_31); -lean_dec(x_6); -x_33 = lean_ctor_get(x_31, 0); -lean_inc(x_33); -lean_dec(x_31); -lean_inc(x_5); -x_34 = l_Lean_isStructure(x_33, 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; lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_33 = lean_ctor_get(x_26, 1); lean_dec(x_33); -if (x_34 == 0) -{ -lean_object* x_35; lean_object* x_36; -lean_dec(x_5); -lean_dec(x_2); -lean_dec(x_1); -x_35 = lean_box(0); -x_36 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_36, 0, x_35); -lean_ctor_set(x_36, 1, x_32); -return x_36; -} -else -{ -lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; lean_object* x_42; size_t x_43; size_t x_44; lean_object* x_45; lean_object* x_46; -x_37 = lean_st_ref_get(x_3, x_32); -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_ctor_get(x_38, 0); +x_34 = lean_ctor_get(x_26, 0); +lean_dec(x_34); +x_35 = l_Lean_Elab_Command_mkState___closed__8; +x_36 = l_Lean_Elab_Command_mkState___closed__11; +lean_ctor_set(x_26, 1, x_36); +lean_ctor_set(x_26, 0, x_35); +x_37 = l___private_Lean_Elab_Command_0__Lean_Elab_Command_runCore___rarg___closed__4; +lean_inc(x_14); +x_38 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_38, 0, x_23); +lean_ctor_set(x_38, 1, x_37); +lean_ctor_set(x_38, 2, x_6); +lean_ctor_set(x_38, 3, x_24); +lean_ctor_set(x_38, 4, x_14); +lean_ctor_set(x_38, 5, x_25); +lean_ctor_set(x_38, 6, x_26); +lean_ctor_set(x_38, 7, x_36); +x_39 = lean_st_mk_ref(x_38, x_9); +x_40 = lean_ctor_get(x_39, 0); lean_inc(x_40); -lean_dec(x_38); -x_41 = 1; -lean_inc(x_5); -x_42 = l_Lean_getStructureFieldsFlattened(x_40, x_5, x_41); -lean_dec(x_40); -x_43 = lean_array_size(x_42); -x_44 = 0; -x_45 = lean_box(0); -x_46 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5(x_1, x_5, x_42, x_43, x_44, x_45, x_2, x_3, x_39); -lean_dec(x_42); -if (lean_obj_tag(x_46) == 0) +x_41 = lean_ctor_get(x_39, 1); +lean_inc(x_41); +lean_dec(x_39); +lean_inc(x_40); +x_42 = lean_apply_3(x_1, x_22, x_40, x_41); +if (lean_obj_tag(x_42) == 0) { -lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_47 = lean_ctor_get(x_46, 1); +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; +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_40, x_44); +lean_dec(x_40); +x_46 = lean_ctor_get(x_45, 0); +lean_inc(x_46); +x_47 = lean_ctor_get(x_45, 1); lean_inc(x_47); -if (lean_is_exclusive(x_46)) { - lean_ctor_release(x_46, 0); - lean_ctor_release(x_46, 1); - x_48 = x_46; -} else { - lean_dec_ref(x_46); - x_48 = lean_box(0); -} -if (lean_is_scalar(x_48)) { - x_49 = lean_alloc_ctor(0, 2, 0); -} else { - x_49 = x_48; -} -lean_ctor_set(x_49, 0, x_45); -lean_ctor_set(x_49, 1, x_47); -return x_49; -} -else -{ -lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; -x_50 = lean_ctor_get(x_46, 0); +lean_dec(x_45); +x_48 = lean_st_ref_take(x_4, 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); -x_51 = lean_ctor_get(x_46, 1); +lean_dec(x_48); +x_51 = lean_ctor_get(x_46, 0); lean_inc(x_51); -if (lean_is_exclusive(x_46)) { - lean_ctor_release(x_46, 0); - lean_ctor_release(x_46, 1); - x_52 = x_46; -} else { - lean_dec_ref(x_46); - x_52 = lean_box(0); -} -if (lean_is_scalar(x_52)) { - x_53 = lean_alloc_ctor(1, 2, 0); -} else { - x_53 = x_52; -} -lean_ctor_set(x_53, 0, x_50); -lean_ctor_set(x_53, 1, x_51); -return x_53; -} -} -} -} -else -{ -lean_object* x_54; lean_object* x_55; -lean_dec(x_2); -lean_dec(x_1); -x_54 = lean_box(0); -x_55 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_55, 0, x_54); -lean_ctor_set(x_55, 1, x_4); -return x_55; -} -} -} -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___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; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; -x_5 = l_Lean_Elab_Command_getRef(x_2, x_3, x_4); -x_6 = lean_ctor_get(x_5, 0); -lean_inc(x_6); -x_7 = lean_ctor_get(x_5, 1); -lean_inc(x_7); -lean_dec(x_5); -x_8 = lean_ctor_get(x_2, 4); -lean_inc(x_8); -lean_inc(x_8); -x_9 = l_Lean_Elab_getBetterRef(x_6, x_8); -lean_dec(x_6); -x_10 = l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1(x_1, x_2, x_3, x_7); -x_11 = !lean_is_exclusive(x_10); -if (x_11 == 0) -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; -x_12 = lean_ctor_get(x_10, 0); -x_13 = lean_ctor_get(x_10, 1); -x_14 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_12, x_8, x_2, x_3, x_13); -lean_dec(x_2); -x_15 = !lean_is_exclusive(x_14); -if (x_15 == 0) -{ -lean_object* x_16; -x_16 = lean_ctor_get(x_14, 0); -lean_ctor_set(x_10, 1, x_16); -lean_ctor_set(x_10, 0, x_9); -lean_ctor_set_tag(x_14, 1); -lean_ctor_set(x_14, 0, x_10); -return x_14; -} -else -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_14, 0); -x_18 = lean_ctor_get(x_14, 1); -lean_inc(x_18); -lean_inc(x_17); -lean_dec(x_14); -lean_ctor_set(x_10, 1, x_17); -lean_ctor_set(x_10, 0, x_9); -x_19 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_19, 0, x_10); -lean_ctor_set(x_19, 1, 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; lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_20 = lean_ctor_get(x_10, 0); -x_21 = lean_ctor_get(x_10, 1); -lean_inc(x_21); -lean_inc(x_20); -lean_dec(x_10); -x_22 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_20, x_8, x_2, x_3, x_21); -lean_dec(x_2); -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -x_24 = lean_ctor_get(x_22, 1); -lean_inc(x_24); -if (lean_is_exclusive(x_22)) { - lean_ctor_release(x_22, 0); - lean_ctor_release(x_22, 1); - x_25 = x_22; -} else { - lean_dec_ref(x_22); - x_25 = lean_box(0); -} -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_9); -lean_ctor_set(x_26, 1, x_23); -if (lean_is_scalar(x_25)) { - x_27 = lean_alloc_ctor(1, 2, 0); -} else { - x_27 = x_25; - lean_ctor_set_tag(x_27, 1); -} -lean_ctor_set(x_27, 0, x_26); -lean_ctor_set(x_27, 1, x_24); -return x_27; -} -} -} -static lean_object* _init_l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("unknown constant '", 18, 18); -return x_1; -} -} -static lean_object* _init_l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9(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_3, x_4); -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; -x_7 = lean_ctor_get(x_5, 0); -x_8 = lean_ctor_get(x_5, 1); -x_9 = lean_ctor_get(x_7, 0); -lean_inc(x_9); -lean_dec(x_7); -lean_inc(x_1); -x_10 = lean_environment_find(x_9, x_1); -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; -lean_free_object(x_5); -x_11 = lean_box(0); -x_12 = l_Lean_Expr_const___override(x_1, x_11); -x_13 = l_Lean_MessageData_ofExpr(x_12); -x_14 = l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9___closed__2; -x_15 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_15, 0, x_14); -lean_ctor_set(x_15, 1, x_13); -x_16 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__8; -x_17 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_17, 0, x_15); -lean_ctor_set(x_17, 1, x_16); -x_18 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__10(x_17, x_2, x_3, x_8); -return x_18; -} -else -{ -lean_object* x_19; -lean_dec(x_2); -lean_dec(x_1); -x_19 = lean_ctor_get(x_10, 0); -lean_inc(x_19); -lean_dec(x_10); -lean_ctor_set(x_5, 0, x_19); -return x_5; -} -} -else -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_20 = lean_ctor_get(x_5, 0); -x_21 = lean_ctor_get(x_5, 1); -lean_inc(x_21); -lean_inc(x_20); -lean_dec(x_5); -x_22 = lean_ctor_get(x_20, 0); -lean_inc(x_22); -lean_dec(x_20); -lean_inc(x_1); -x_23 = lean_environment_find(x_22, x_1); -if (lean_obj_tag(x_23) == 0) -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_24 = lean_box(0); -x_25 = l_Lean_Expr_const___override(x_1, x_24); -x_26 = l_Lean_MessageData_ofExpr(x_25); -x_27 = l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9___closed__2; -x_28 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_28, 0, x_27); -lean_ctor_set(x_28, 1, x_26); -x_29 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__8; -x_30 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_30, 0, x_28); -lean_ctor_set(x_30, 1, x_29); -x_31 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__10(x_30, x_2, x_3, x_21); -return x_31; -} -else -{ -lean_object* x_32; lean_object* x_33; -lean_dec(x_2); -lean_dec(x_1); -x_32 = lean_ctor_get(x_23, 0); -lean_inc(x_32); -lean_dec(x_23); -x_33 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_33, 0, x_32); -lean_ctor_set(x_33, 1, x_21); -return x_33; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_mkConstWithLevelParams___at_Lean_Elab_Command_expandDeclId___spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -lean_object* x_5; -lean_inc(x_1); -x_5 = l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9(x_1, x_2, x_3, x_4); -if (lean_obj_tag(x_5) == 0) -{ -uint8_t x_6; -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; -x_7 = lean_ctor_get(x_5, 0); -x_8 = l_Lean_ConstantInfo_levelParams(x_7); -lean_dec(x_7); -x_9 = lean_box(0); -x_10 = l_List_mapTR_loop___at_Lean_mkConstWithLevelParams___spec__1(x_8, x_9); -x_11 = l_Lean_Expr_const___override(x_1, 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; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_12 = lean_ctor_get(x_5, 0); -x_13 = lean_ctor_get(x_5, 1); -lean_inc(x_13); -lean_inc(x_12); -lean_dec(x_5); -x_14 = l_Lean_ConstantInfo_levelParams(x_12); -lean_dec(x_12); -x_15 = lean_box(0); -x_16 = l_List_mapTR_loop___at_Lean_mkConstWithLevelParams___spec__1(x_14, x_15); -x_17 = l_Lean_Expr_const___override(x_1, x_16); -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_17); -lean_ctor_set(x_18, 1, x_13); -return x_18; -} -} -else -{ -uint8_t x_19; -lean_dec(x_1); -x_19 = !lean_is_exclusive(x_5); -if (x_19 == 0) -{ -return x_5; -} -else -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_5, 0); -x_21 = lean_ctor_get(x_5, 1); -lean_inc(x_21); -lean_inc(x_20); -lean_dec(x_5); -x_22 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_22, 0, x_20); -lean_ctor_set(x_22, 1, x_21); -return x_22; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoTree___at_Lean_Elab_Command_expandDeclId___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; uint8_t x_8; -x_5 = lean_st_ref_get(x_3, x_4); -x_6 = lean_ctor_get(x_5, 0); -lean_inc(x_6); -x_7 = lean_ctor_get(x_6, 6); -lean_inc(x_7); -lean_dec(x_6); -x_8 = lean_ctor_get_uint8(x_7, sizeof(void*)*2); -lean_dec(x_7); -if (x_8 == 0) -{ -uint8_t x_9; -lean_dec(x_1); -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); -lean_dec(x_10); -x_11 = lean_box(0); -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, 1); -lean_inc(x_12); -lean_dec(x_5); -x_13 = lean_box(0); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_13); -lean_ctor_set(x_14, 1, x_12); -return x_14; -} -} -else -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; -x_15 = lean_ctor_get(x_5, 1); -lean_inc(x_15); -lean_dec(x_5); -x_16 = lean_st_ref_take(x_3, x_15); -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_17, 6); -lean_inc(x_18); -x_19 = lean_ctor_get(x_16, 1); -lean_inc(x_19); -lean_dec(x_16); -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, 6); -lean_dec(x_21); -x_22 = !lean_is_exclusive(x_18); -if (x_22 == 0) -{ -lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; -x_23 = lean_ctor_get(x_18, 1); -x_24 = l_Lean_PersistentArray_push___rarg(x_23, x_1); -lean_ctor_set(x_18, 1, x_24); -x_25 = lean_st_ref_set(x_3, x_17, x_19); -x_26 = !lean_is_exclusive(x_25); -if (x_26 == 0) +x_52 = lean_ctor_get(x_46, 1); +lean_inc(x_52); +x_53 = lean_ctor_get(x_46, 3); +lean_inc(x_53); +x_54 = lean_ctor_get(x_46, 5); +lean_inc(x_54); +x_55 = lean_ctor_get(x_46, 6); +lean_inc(x_55); +x_56 = lean_ctor_get(x_46, 7); +lean_inc(x_56); +lean_dec(x_46); +x_57 = !lean_is_exclusive(x_49); +if (x_57 == 0) { -lean_object* x_27; lean_object* x_28; -x_27 = lean_ctor_get(x_25, 0); -lean_dec(x_27); -x_28 = lean_box(0); -lean_ctor_set(x_25, 0, x_28); -return x_25; -} -else +lean_object* x_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_49, 3); +x_59 = lean_ctor_get(x_49, 2); +lean_dec(x_59); +x_60 = lean_ctor_get(x_49, 1); +lean_dec(x_60); +x_61 = lean_ctor_get(x_49, 0); +lean_dec(x_61); +x_62 = l_Lean_PersistentArray_append___rarg(x_58, x_56); +lean_dec(x_56); +lean_ctor_set(x_49, 3, x_62); +lean_ctor_set(x_49, 2, x_54); +lean_ctor_set(x_49, 1, x_53); +lean_ctor_set(x_49, 0, x_51); +x_63 = lean_st_ref_set(x_4, x_49, x_50); +if (x_2 == 0) { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_25, 1); -lean_inc(x_29); -lean_dec(x_25); -x_30 = lean_box(0); -x_31 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_31, 0, x_30); -lean_ctor_set(x_31, 1, x_29); -return x_31; -} +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 = lean_box(0); +x_66 = l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___lambda__1(x_52, x_55, x_43, x_65, x_3, x_4, x_64); +lean_dec(x_55); +return x_66; } else { -uint8_t x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_32 = lean_ctor_get_uint8(x_18, sizeof(void*)*2); -x_33 = lean_ctor_get(x_18, 0); -x_34 = lean_ctor_get(x_18, 1); -lean_inc(x_34); -lean_inc(x_33); -lean_dec(x_18); -x_35 = l_Lean_PersistentArray_push___rarg(x_34, x_1); -x_36 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_36, 0, x_33); -lean_ctor_set(x_36, 1, x_35); -lean_ctor_set_uint8(x_36, sizeof(void*)*2, x_32); -lean_ctor_set(x_17, 6, x_36); -x_37 = lean_st_ref_set(x_3, x_17, x_19); -x_38 = lean_ctor_get(x_37, 1); -lean_inc(x_38); -if (lean_is_exclusive(x_37)) { - lean_ctor_release(x_37, 0); - lean_ctor_release(x_37, 1); - x_39 = x_37; -} else { - lean_dec_ref(x_37); - x_39 = lean_box(0); -} -x_40 = lean_box(0); -if (lean_is_scalar(x_39)) { - x_41 = lean_alloc_ctor(0, 2, 0); -} else { - x_41 = x_39; -} -lean_ctor_set(x_41, 0, x_40); -lean_ctor_set(x_41, 1, x_38); -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; uint8_t x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_42 = lean_ctor_get(x_17, 0); -x_43 = lean_ctor_get(x_17, 1); -x_44 = lean_ctor_get(x_17, 2); -x_45 = lean_ctor_get(x_17, 3); -x_46 = lean_ctor_get(x_17, 4); -x_47 = lean_ctor_get(x_17, 5); -x_48 = lean_ctor_get(x_17, 7); -lean_inc(x_48); -lean_inc(x_47); -lean_inc(x_46); -lean_inc(x_45); -lean_inc(x_44); -lean_inc(x_43); -lean_inc(x_42); -lean_dec(x_17); -x_49 = lean_ctor_get_uint8(x_18, sizeof(void*)*2); -x_50 = lean_ctor_get(x_18, 0); -lean_inc(x_50); -x_51 = lean_ctor_get(x_18, 1); -lean_inc(x_51); -if (lean_is_exclusive(x_18)) { - lean_ctor_release(x_18, 0); - lean_ctor_release(x_18, 1); - x_52 = x_18; -} else { - lean_dec_ref(x_18); - x_52 = lean_box(0); -} -x_53 = l_Lean_PersistentArray_push___rarg(x_51, x_1); -if (lean_is_scalar(x_52)) { - x_54 = lean_alloc_ctor(0, 2, 1); -} else { - x_54 = x_52; -} -lean_ctor_set(x_54, 0, x_50); -lean_ctor_set(x_54, 1, x_53); -lean_ctor_set_uint8(x_54, sizeof(void*)*2, x_49); -x_55 = lean_alloc_ctor(0, 8, 0); -lean_ctor_set(x_55, 0, x_42); -lean_ctor_set(x_55, 1, x_43); -lean_ctor_set(x_55, 2, x_44); -lean_ctor_set(x_55, 3, x_45); -lean_ctor_set(x_55, 4, x_46); -lean_ctor_set(x_55, 5, x_47); -lean_ctor_set(x_55, 6, x_54); -lean_ctor_set(x_55, 7, x_48); -x_56 = lean_st_ref_set(x_3, x_55, x_19); -x_57 = lean_ctor_get(x_56, 1); -lean_inc(x_57); -if (lean_is_exclusive(x_56)) { - lean_ctor_release(x_56, 0); - lean_ctor_release(x_56, 1); - x_58 = x_56; -} else { - lean_dec_ref(x_56); - x_58 = lean_box(0); -} -x_59 = lean_box(0); -if (lean_is_scalar(x_58)) { - x_60 = lean_alloc_ctor(0, 2, 0); -} else { - x_60 = x_58; -} -lean_ctor_set(x_60, 0, x_59); -lean_ctor_set(x_60, 1, x_57); -return x_60; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_expandDeclId___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; uint8_t x_8; -x_5 = lean_st_ref_get(x_3, x_4); -x_6 = lean_ctor_get(x_5, 0); -lean_inc(x_6); -x_7 = lean_ctor_get(x_6, 6); -lean_inc(x_7); -lean_dec(x_6); -x_8 = lean_ctor_get_uint8(x_7, sizeof(void*)*2); -lean_dec(x_7); -if (x_8 == 0) -{ -uint8_t x_9; -lean_dec(x_1); -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); -lean_dec(x_10); -x_11 = lean_box(0); -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, 1); -lean_inc(x_12); -lean_dec(x_5); -x_13 = lean_box(0); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_13); -lean_ctor_set(x_14, 1, x_12); -return x_14; -} -} -else -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_15 = lean_ctor_get(x_5, 1); -lean_inc(x_15); -lean_dec(x_5); -x_16 = l_Lean_Elab_Command_mkState___closed__11; -x_17 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_17, 0, x_1); -lean_ctor_set(x_17, 1, x_16); -x_18 = l_Lean_Elab_pushInfoTree___at_Lean_Elab_Command_expandDeclId___spec__12(x_17, x_2, x_3, x_15); -return x_18; -} -} -} -static lean_object* _init_l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__1___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("a non-private declaration '", 27, 27); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__1___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__1___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___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) { -_start: -{ -lean_object* x_7; -x_7 = lean_private_to_user_name(x_1); -if (lean_obj_tag(x_7) == 0) -{ -lean_object* x_8; lean_object* x_9; -lean_dec(x_4); -lean_dec(x_2); -x_8 = lean_box(0); -x_9 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_9, 0, x_8); -lean_ctor_set(x_9, 1, x_6); -return x_9; -} -else -{ -uint8_t x_10; -x_10 = !lean_is_exclusive(x_7); -if (x_10 == 0) -{ -lean_object* x_11; uint8_t x_12; -x_11 = lean_ctor_get(x_7, 0); -x_12 = l_Lean_Environment_contains(x_2, x_11); -if (x_12 == 0) -{ -lean_object* x_13; lean_object* x_14; -lean_free_object(x_7); -lean_dec(x_11); -lean_dec(x_4); -x_13 = lean_box(0); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_13); -lean_ctor_set(x_14, 1, x_6); -return x_14; -} -else -{ -lean_object* x_15; uint8_t x_16; -x_15 = l_Lean_Elab_Command_getRef(x_4, x_5, x_6); -x_16 = !lean_is_exclusive(x_15); -if (x_16 == 0) -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_15, 0); -x_18 = lean_ctor_get(x_15, 1); -lean_inc(x_4); -lean_inc(x_11); -x_19 = l_Lean_mkConstWithLevelParams___at_Lean_Elab_Command_expandDeclId___spec__8(x_11, x_4, x_5, 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; uint8_t x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_19, 1); -lean_inc(x_21); -lean_dec(x_19); -x_22 = lean_box(0); -lean_ctor_set(x_15, 1, x_17); -lean_ctor_set(x_15, 0, x_22); -x_23 = lean_box(0); -x_24 = l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1___closed__2; -x_25 = 0; -x_26 = lean_alloc_ctor(0, 4, 1); -lean_ctor_set(x_26, 0, x_15); -lean_ctor_set(x_26, 1, x_24); -lean_ctor_set(x_26, 2, x_23); -lean_ctor_set(x_26, 3, x_20); -lean_ctor_set_uint8(x_26, sizeof(void*)*4, x_25); -lean_ctor_set(x_7, 0, x_26); -x_27 = l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_expandDeclId___spec__11(x_7, x_4, x_5, x_21); -x_28 = !lean_is_exclusive(x_27); -if (x_28 == 0) -{ -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_29 = lean_ctor_get(x_27, 1); -x_30 = lean_ctor_get(x_27, 0); -lean_dec(x_30); -x_31 = l_Lean_MessageData_ofName(x_11); -x_32 = l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__1___closed__2; -lean_ctor_set_tag(x_27, 7); -lean_ctor_set(x_27, 1, x_31); -lean_ctor_set(x_27, 0, x_32); -x_33 = l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_addUnivLevel___spec__1___closed__4; -x_34 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_34, 0, x_27); -lean_ctor_set(x_34, 1, x_33); -x_35 = l_Lean_throwError___at___private_Lean_Elab_Command_0__Lean_Elab_Command_elabCommandUsing___spec__1(x_34, x_4, x_5, x_29); -return x_35; -} -else -{ -lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_36 = lean_ctor_get(x_27, 1); -lean_inc(x_36); -lean_dec(x_27); -x_37 = l_Lean_MessageData_ofName(x_11); -x_38 = l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__1___closed__2; -x_39 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_39, 0, x_38); -lean_ctor_set(x_39, 1, x_37); -x_40 = l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_addUnivLevel___spec__1___closed__4; -x_41 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_41, 0, x_39); -lean_ctor_set(x_41, 1, x_40); -x_42 = l_Lean_throwError___at___private_Lean_Elab_Command_0__Lean_Elab_Command_elabCommandUsing___spec__1(x_41, x_4, x_5, x_36); -return x_42; -} -} -else -{ -uint8_t x_43; -lean_free_object(x_15); -lean_dec(x_17); -lean_free_object(x_7); -lean_dec(x_11); -lean_dec(x_4); -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 -{ -lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_47 = lean_ctor_get(x_15, 0); -x_48 = lean_ctor_get(x_15, 1); -lean_inc(x_48); -lean_inc(x_47); -lean_dec(x_15); -lean_inc(x_4); -lean_inc(x_11); -x_49 = l_Lean_mkConstWithLevelParams___at_Lean_Elab_Command_expandDeclId___spec__8(x_11, x_4, x_5, x_48); -if (lean_obj_tag(x_49) == 0) -{ -lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; 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; -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_box(0); -x_53 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_53, 0, x_52); -lean_ctor_set(x_53, 1, x_47); -x_54 = lean_box(0); -x_55 = l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1___closed__2; -x_56 = 0; -x_57 = lean_alloc_ctor(0, 4, 1); -lean_ctor_set(x_57, 0, x_53); -lean_ctor_set(x_57, 1, x_55); -lean_ctor_set(x_57, 2, x_54); -lean_ctor_set(x_57, 3, x_50); -lean_ctor_set_uint8(x_57, sizeof(void*)*4, x_56); -lean_ctor_set(x_7, 0, x_57); -x_58 = l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_expandDeclId___spec__11(x_7, x_4, x_5, x_51); -x_59 = lean_ctor_get(x_58, 1); -lean_inc(x_59); -if (lean_is_exclusive(x_58)) { - lean_ctor_release(x_58, 0); - lean_ctor_release(x_58, 1); - x_60 = x_58; -} else { - lean_dec_ref(x_58); - x_60 = lean_box(0); -} -x_61 = l_Lean_MessageData_ofName(x_11); -x_62 = l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__1___closed__2; -if (lean_is_scalar(x_60)) { - x_63 = lean_alloc_ctor(7, 2, 0); -} else { - x_63 = x_60; - lean_ctor_set_tag(x_63, 7); -} -lean_ctor_set(x_63, 0, x_62); -lean_ctor_set(x_63, 1, x_61); -x_64 = l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_addUnivLevel___spec__1___closed__4; -x_65 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_65, 0, x_63); -lean_ctor_set(x_65, 1, x_64); -x_66 = l_Lean_throwError___at___private_Lean_Elab_Command_0__Lean_Elab_Command_elabCommandUsing___spec__1(x_65, x_4, x_5, x_59); -return x_66; -} -else -{ -lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; -lean_dec(x_47); -lean_free_object(x_7); -lean_dec(x_11); -lean_dec(x_4); -x_67 = lean_ctor_get(x_49, 0); +lean_object* x_67; lean_object* x_68; size_t x_69; size_t x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; +x_67 = lean_ctor_get(x_63, 1); lean_inc(x_67); -x_68 = lean_ctor_get(x_49, 1); -lean_inc(x_68); -if (lean_is_exclusive(x_49)) { - lean_ctor_release(x_49, 0); - lean_ctor_release(x_49, 1); - x_69 = x_49; -} else { - lean_dec_ref(x_49); - x_69 = lean_box(0); -} -if (lean_is_scalar(x_69)) { - x_70 = lean_alloc_ctor(1, 2, 0); -} else { - x_70 = x_69; -} -lean_ctor_set(x_70, 0, x_67); -lean_ctor_set(x_70, 1, x_68); -return x_70; -} -} -} -} -else -{ -lean_object* x_71; uint8_t x_72; -x_71 = lean_ctor_get(x_7, 0); -lean_inc(x_71); -lean_dec(x_7); -x_72 = l_Lean_Environment_contains(x_2, x_71); -if (x_72 == 0) -{ -lean_object* x_73; lean_object* x_74; -lean_dec(x_71); -lean_dec(x_4); -x_73 = lean_box(0); -x_74 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_74, 0, x_73); -lean_ctor_set(x_74, 1, x_6); -return x_74; -} -else -{ -lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; -x_75 = l_Lean_Elab_Command_getRef(x_4, x_5, x_6); -x_76 = lean_ctor_get(x_75, 0); -lean_inc(x_76); -x_77 = lean_ctor_get(x_75, 1); -lean_inc(x_77); -if (lean_is_exclusive(x_75)) { - lean_ctor_release(x_75, 0); - lean_ctor_release(x_75, 1); - x_78 = x_75; -} else { - lean_dec_ref(x_75); - x_78 = lean_box(0); -} -lean_inc(x_4); -lean_inc(x_71); -x_79 = l_Lean_mkConstWithLevelParams___at_Lean_Elab_Command_expandDeclId___spec__8(x_71, x_4, x_5, 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; lean_object* x_85; uint8_t x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; -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_box(0); -if (lean_is_scalar(x_78)) { - x_83 = lean_alloc_ctor(0, 2, 0); -} else { - x_83 = x_78; -} -lean_ctor_set(x_83, 0, x_82); -lean_ctor_set(x_83, 1, x_76); -x_84 = lean_box(0); -x_85 = l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1___closed__2; -x_86 = 0; -x_87 = lean_alloc_ctor(0, 4, 1); -lean_ctor_set(x_87, 0, x_83); -lean_ctor_set(x_87, 1, x_85); -lean_ctor_set(x_87, 2, x_84); -lean_ctor_set(x_87, 3, x_80); -lean_ctor_set_uint8(x_87, sizeof(void*)*4, x_86); -x_88 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_88, 0, x_87); -x_89 = l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_expandDeclId___spec__11(x_88, x_4, x_5, x_81); -x_90 = lean_ctor_get(x_89, 1); -lean_inc(x_90); -if (lean_is_exclusive(x_89)) { - lean_ctor_release(x_89, 0); - lean_ctor_release(x_89, 1); - x_91 = x_89; -} else { - lean_dec_ref(x_89); - x_91 = lean_box(0); -} -x_92 = l_Lean_MessageData_ofName(x_71); -x_93 = l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__1___closed__2; -if (lean_is_scalar(x_91)) { - x_94 = lean_alloc_ctor(7, 2, 0); -} else { - x_94 = x_91; - lean_ctor_set_tag(x_94, 7); -} -lean_ctor_set(x_94, 0, x_93); -lean_ctor_set(x_94, 1, x_92); -x_95 = l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_addUnivLevel___spec__1___closed__4; -x_96 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_96, 0, x_94); -lean_ctor_set(x_96, 1, x_95); -x_97 = l_Lean_throwError___at___private_Lean_Elab_Command_0__Lean_Elab_Command_elabCommandUsing___spec__1(x_96, x_4, x_5, x_90); -return x_97; -} -else -{ -lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; -lean_dec(x_78); -lean_dec(x_76); -lean_dec(x_71); -lean_dec(x_4); -x_98 = lean_ctor_get(x_79, 0); -lean_inc(x_98); -x_99 = lean_ctor_get(x_79, 1); -lean_inc(x_99); -if (lean_is_exclusive(x_79)) { - lean_ctor_release(x_79, 0); - lean_ctor_release(x_79, 1); - x_100 = x_79; -} else { - lean_dec_ref(x_79); - x_100 = lean_box(0); -} -if (lean_is_scalar(x_100)) { - x_101 = lean_alloc_ctor(1, 2, 0); -} else { - x_101 = x_100; -} -lean_ctor_set(x_101, 0, x_98); -lean_ctor_set(x_101, 1, x_99); -return x_101; -} -} -} -} -} -} -static lean_object* _init_l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__2___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("a private declaration '", 23, 23); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__2___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__2___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___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; uint8_t x_8; -lean_inc(x_1); -lean_inc(x_2); -x_7 = l_Lean_mkPrivateName(x_2, x_1); -lean_inc(x_2); -x_8 = l_Lean_Environment_contains(x_2, x_7); -if (x_8 == 0) -{ -lean_object* x_9; lean_object* x_10; -lean_dec(x_7); -x_9 = lean_box(0); -x_10 = l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__1(x_1, x_2, x_9, x_4, x_5, x_6); -return x_10; -} -else -{ -lean_object* x_11; uint8_t x_12; -lean_dec(x_2); -x_11 = l_Lean_Elab_Command_getRef(x_4, x_5, 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; -x_13 = lean_ctor_get(x_11, 0); -x_14 = lean_ctor_get(x_11, 1); -lean_inc(x_4); -x_15 = l_Lean_mkConstWithLevelParams___at_Lean_Elab_Command_expandDeclId___spec__8(x_7, x_4, x_5, 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; uint8_t x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; -x_16 = lean_ctor_get(x_15, 0); -lean_inc(x_16); -x_17 = lean_ctor_get(x_15, 1); -lean_inc(x_17); -lean_dec(x_15); -x_18 = lean_box(0); -lean_ctor_set(x_11, 1, x_13); -lean_ctor_set(x_11, 0, x_18); -x_19 = lean_box(0); -x_20 = l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1___closed__2; -x_21 = 0; -x_22 = lean_alloc_ctor(0, 4, 1); -lean_ctor_set(x_22, 0, x_11); -lean_ctor_set(x_22, 1, x_20); -lean_ctor_set(x_22, 2, x_19); -lean_ctor_set(x_22, 3, x_16); -lean_ctor_set_uint8(x_22, sizeof(void*)*4, x_21); -x_23 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_23, 0, x_22); -x_24 = l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_expandDeclId___spec__11(x_23, x_4, x_5, x_17); -x_25 = !lean_is_exclusive(x_24); -if (x_25 == 0) -{ -lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; -x_26 = lean_ctor_get(x_24, 1); -x_27 = lean_ctor_get(x_24, 0); -lean_dec(x_27); -x_28 = l_Lean_MessageData_ofName(x_1); -x_29 = l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__2___closed__2; -lean_ctor_set_tag(x_24, 7); -lean_ctor_set(x_24, 1, x_28); -lean_ctor_set(x_24, 0, x_29); -x_30 = l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_addUnivLevel___spec__1___closed__4; -x_31 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_31, 0, x_24); -lean_ctor_set(x_31, 1, x_30); -x_32 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_31, x_4, x_5, x_26); -x_33 = !lean_is_exclusive(x_32); -if (x_33 == 0) -{ -return x_32; -} -else -{ -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_32, 0); -x_35 = lean_ctor_get(x_32, 1); -lean_inc(x_35); -lean_inc(x_34); -lean_dec(x_32); -x_36 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_36, 0, x_34); -lean_ctor_set(x_36, 1, x_35); -return x_36; -} -} -else -{ -lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_37 = lean_ctor_get(x_24, 1); -lean_inc(x_37); -lean_dec(x_24); -x_38 = l_Lean_MessageData_ofName(x_1); -x_39 = l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__2___closed__2; -x_40 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_40, 0, x_39); -lean_ctor_set(x_40, 1, x_38); -x_41 = l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_addUnivLevel___spec__1___closed__4; -x_42 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_42, 0, x_40); -lean_ctor_set(x_42, 1, x_41); -x_43 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_42, x_4, x_5, x_37); -x_44 = lean_ctor_get(x_43, 0); -lean_inc(x_44); -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); -} -if (lean_is_scalar(x_46)) { - x_47 = lean_alloc_ctor(1, 2, 0); -} else { - x_47 = x_46; -} -lean_ctor_set(x_47, 0, x_44); -lean_ctor_set(x_47, 1, x_45); -return x_47; -} -} -else -{ -uint8_t x_48; -lean_free_object(x_11); -lean_dec(x_13); -lean_dec(x_4); -lean_dec(x_1); -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; -} -} -} -else -{ -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); -lean_inc(x_4); -x_54 = l_Lean_mkConstWithLevelParams___at_Lean_Elab_Command_expandDeclId___spec__8(x_7, x_4, x_5, x_53); -if (lean_obj_tag(x_54) == 0) -{ -lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; uint8_t x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; -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_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_52); -x_59 = lean_box(0); -x_60 = l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1___closed__2; -x_61 = 0; -x_62 = lean_alloc_ctor(0, 4, 1); -lean_ctor_set(x_62, 0, x_58); -lean_ctor_set(x_62, 1, x_60); -lean_ctor_set(x_62, 2, x_59); -lean_ctor_set(x_62, 3, x_55); -lean_ctor_set_uint8(x_62, sizeof(void*)*4, x_61); -x_63 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_63, 0, x_62); -x_64 = l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_expandDeclId___spec__11(x_63, x_4, x_5, x_56); -x_65 = lean_ctor_get(x_64, 1); -lean_inc(x_65); -if (lean_is_exclusive(x_64)) { - lean_ctor_release(x_64, 0); - lean_ctor_release(x_64, 1); - x_66 = x_64; -} else { - lean_dec_ref(x_64); - x_66 = lean_box(0); -} -x_67 = l_Lean_MessageData_ofName(x_1); -x_68 = l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__2___closed__2; -if (lean_is_scalar(x_66)) { - x_69 = lean_alloc_ctor(7, 2, 0); -} else { - x_69 = x_66; - lean_ctor_set_tag(x_69, 7); -} -lean_ctor_set(x_69, 0, x_68); -lean_ctor_set(x_69, 1, x_67); -x_70 = l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_addUnivLevel___spec__1___closed__4; -x_71 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_71, 0, x_69); -lean_ctor_set(x_71, 1, x_70); -x_72 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_71, x_4, x_5, x_65); -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; -} -else -{ -lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; -lean_dec(x_52); -lean_dec(x_4); -lean_dec(x_1); -x_77 = lean_ctor_get(x_54, 0); -lean_inc(x_77); -x_78 = lean_ctor_get(x_54, 1); -lean_inc(x_78); -if (lean_is_exclusive(x_54)) { - lean_ctor_release(x_54, 0); - lean_ctor_release(x_54, 1); - x_79 = x_54; -} else { - lean_dec_ref(x_54); - 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; -} -} -} -} -} -static lean_object* _init_l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__3___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("' is a reserved name", 20, 20); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__3___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__3___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___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: -{ -uint8_t x_7; -lean_inc(x_1); -lean_inc(x_2); -x_7 = l_Lean_isReservedName(x_2, x_1); -if (x_7 == 0) -{ -lean_object* x_8; lean_object* x_9; -x_8 = lean_box(0); -x_9 = l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__2(x_1, x_2, x_8, x_4, x_5, x_6); -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; uint8_t x_16; -lean_dec(x_2); -x_10 = l_Lean_MessageData_ofName(x_1); -x_11 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__8; -x_12 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_12, 0, x_11); -lean_ctor_set(x_12, 1, x_10); -x_13 = l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__3___closed__2; -x_14 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_14, 0, x_12); -lean_ctor_set(x_14, 1, x_13); -x_15 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_14, x_4, x_5, x_6); -x_16 = !lean_is_exclusive(x_15); -if (x_16 == 0) -{ -return x_15; -} -else -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_15, 0); -x_18 = lean_ctor_get(x_15, 1); -lean_inc(x_18); -lean_inc(x_17); -lean_dec(x_15); -x_19 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_19, 0, x_17); -lean_ctor_set(x_19, 1, x_18); -return x_19; -} -} -} -} -static lean_object* _init_l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("private declaration '", 21, 21); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___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; -x_5 = lean_st_ref_get(x_3, x_4); -x_6 = !lean_is_exclusive(x_5); -if (x_6 == 0) -{ -lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; -x_7 = lean_ctor_get(x_5, 0); -x_8 = lean_ctor_get(x_5, 1); -x_9 = lean_ctor_get(x_7, 0); -lean_inc(x_9); -lean_dec(x_7); -lean_inc(x_9); -x_10 = l_Lean_Environment_contains(x_9, x_1); -if (x_10 == 0) -{ -lean_object* x_11; lean_object* x_12; -lean_free_object(x_5); -x_11 = lean_box(0); -x_12 = l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__3(x_1, x_9, x_11, x_2, x_3, x_8); -return x_12; -} -else -{ -lean_object* x_13; uint8_t x_14; -lean_dec(x_9); -x_13 = l_Lean_Elab_Command_getRef(x_2, x_3, x_8); -x_14 = !lean_is_exclusive(x_13); -if (x_14 == 0) -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = lean_ctor_get(x_13, 0); -x_16 = lean_ctor_get(x_13, 1); -lean_inc(x_2); -lean_inc(x_1); -x_17 = l_Lean_mkConstWithLevelParams___at_Lean_Elab_Command_expandDeclId___spec__8(x_1, x_2, x_3, x_16); -if (lean_obj_tag(x_17) == 0) -{ -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_17, 1); -lean_inc(x_19); -lean_dec(x_17); -x_20 = lean_box(0); -lean_ctor_set(x_13, 1, x_15); -lean_ctor_set(x_13, 0, x_20); -x_21 = lean_box(0); -x_22 = l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1___closed__2; -x_23 = 0; -x_24 = lean_alloc_ctor(0, 4, 1); -lean_ctor_set(x_24, 0, x_13); -lean_ctor_set(x_24, 1, x_22); -lean_ctor_set(x_24, 2, x_21); -lean_ctor_set(x_24, 3, x_18); -lean_ctor_set_uint8(x_24, sizeof(void*)*4, x_23); -x_25 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_25, 0, x_24); -x_26 = l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_expandDeclId___spec__11(x_25, x_2, x_3, x_19); -x_27 = !lean_is_exclusive(x_26); -if (x_27 == 0) -{ -lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_28 = lean_ctor_get(x_26, 1); -x_29 = lean_ctor_get(x_26, 0); -lean_dec(x_29); -lean_inc(x_1); -x_30 = lean_private_to_user_name(x_1); -if (lean_obj_tag(x_30) == 0) -{ -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; -x_31 = l_Lean_MessageData_ofName(x_1); -x_32 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__8; -lean_ctor_set_tag(x_26, 7); -lean_ctor_set(x_26, 1, x_31); -lean_ctor_set(x_26, 0, x_32); -x_33 = l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_addUnivLevel___spec__1___closed__4; -lean_ctor_set_tag(x_5, 7); -lean_ctor_set(x_5, 1, x_33); -lean_ctor_set(x_5, 0, x_26); -x_34 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_5, x_2, x_3, x_28); -x_35 = !lean_is_exclusive(x_34); -if (x_35 == 0) -{ -return x_34; -} -else -{ -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_34, 0); -x_37 = lean_ctor_get(x_34, 1); -lean_inc(x_37); -lean_inc(x_36); -lean_dec(x_34); -x_38 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -return x_38; -} -} -else -{ -lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; -lean_dec(x_1); -x_39 = lean_ctor_get(x_30, 0); -lean_inc(x_39); -lean_dec(x_30); -x_40 = l_Lean_MessageData_ofName(x_39); -x_41 = l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___closed__2; -lean_ctor_set_tag(x_26, 7); -lean_ctor_set(x_26, 1, x_40); -lean_ctor_set(x_26, 0, x_41); -x_42 = l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_addUnivLevel___spec__1___closed__4; -lean_ctor_set_tag(x_5, 7); -lean_ctor_set(x_5, 1, x_42); -lean_ctor_set(x_5, 0, x_26); -x_43 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_5, x_2, x_3, x_28); -x_44 = !lean_is_exclusive(x_43); -if (x_44 == 0) -{ -return x_43; -} -else -{ -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_43, 0); -x_46 = lean_ctor_get(x_43, 1); -lean_inc(x_46); -lean_inc(x_45); -lean_dec(x_43); -x_47 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_47, 0, x_45); -lean_ctor_set(x_47, 1, x_46); -return x_47; -} -} -} -else -{ -lean_object* x_48; lean_object* x_49; -x_48 = lean_ctor_get(x_26, 1); -lean_inc(x_48); -lean_dec(x_26); -lean_inc(x_1); -x_49 = lean_private_to_user_name(x_1); -if (lean_obj_tag(x_49) == 0) -{ -lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; -x_50 = l_Lean_MessageData_ofName(x_1); -x_51 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__8; -x_52 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_52, 0, x_51); -lean_ctor_set(x_52, 1, x_50); -x_53 = l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_addUnivLevel___spec__1___closed__4; -lean_ctor_set_tag(x_5, 7); -lean_ctor_set(x_5, 1, x_53); -lean_ctor_set(x_5, 0, x_52); -x_54 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_5, x_2, x_3, x_48); -x_55 = lean_ctor_get(x_54, 0); -lean_inc(x_55); -x_56 = lean_ctor_get(x_54, 1); -lean_inc(x_56); -if (lean_is_exclusive(x_54)) { - lean_ctor_release(x_54, 0); - lean_ctor_release(x_54, 1); - x_57 = x_54; -} else { - lean_dec_ref(x_54); - x_57 = lean_box(0); -} -if (lean_is_scalar(x_57)) { - x_58 = lean_alloc_ctor(1, 2, 0); -} else { - x_58 = x_57; -} -lean_ctor_set(x_58, 0, x_55); -lean_ctor_set(x_58, 1, x_56); -return x_58; -} -else -{ -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_1); -x_59 = lean_ctor_get(x_49, 0); -lean_inc(x_59); -lean_dec(x_49); -x_60 = l_Lean_MessageData_ofName(x_59); -x_61 = l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___closed__2; -x_62 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_62, 0, x_61); -lean_ctor_set(x_62, 1, x_60); -x_63 = l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_addUnivLevel___spec__1___closed__4; -lean_ctor_set_tag(x_5, 7); -lean_ctor_set(x_5, 1, x_63); -lean_ctor_set(x_5, 0, x_62); -x_64 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_5, x_2, x_3, x_48); -x_65 = lean_ctor_get(x_64, 0); -lean_inc(x_65); -x_66 = lean_ctor_get(x_64, 1); -lean_inc(x_66); -if (lean_is_exclusive(x_64)) { - lean_ctor_release(x_64, 0); - lean_ctor_release(x_64, 1); - x_67 = x_64; -} else { - lean_dec_ref(x_64); - x_67 = lean_box(0); -} -if (lean_is_scalar(x_67)) { - x_68 = lean_alloc_ctor(1, 2, 0); -} else { - x_68 = x_67; -} -lean_ctor_set(x_68, 0, x_65); -lean_ctor_set(x_68, 1, x_66); -return x_68; -} -} -} -else -{ -uint8_t x_69; -lean_free_object(x_13); -lean_dec(x_15); -lean_free_object(x_5); -lean_dec(x_2); -lean_dec(x_1); -x_69 = !lean_is_exclusive(x_17); -if (x_69 == 0) -{ -return x_17; -} -else -{ -lean_object* x_70; lean_object* x_71; lean_object* x_72; -x_70 = lean_ctor_get(x_17, 0); -x_71 = lean_ctor_get(x_17, 1); -lean_inc(x_71); -lean_inc(x_70); -lean_dec(x_17); -x_72 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_72, 0, x_70); -lean_ctor_set(x_72, 1, x_71); -return x_72; -} -} -} -else -{ -lean_object* x_73; lean_object* x_74; lean_object* x_75; -x_73 = lean_ctor_get(x_13, 0); -x_74 = lean_ctor_get(x_13, 1); -lean_inc(x_74); -lean_inc(x_73); -lean_dec(x_13); -lean_inc(x_2); -lean_inc(x_1); -x_75 = l_Lean_mkConstWithLevelParams___at_Lean_Elab_Command_expandDeclId___spec__8(x_1, x_2, x_3, x_74); -if (lean_obj_tag(x_75) == 0) -{ -lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; uint8_t x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; -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_box(0); -x_79 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_79, 0, x_78); -lean_ctor_set(x_79, 1, x_73); -x_80 = lean_box(0); -x_81 = l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1___closed__2; -x_82 = 0; -x_83 = lean_alloc_ctor(0, 4, 1); -lean_ctor_set(x_83, 0, x_79); -lean_ctor_set(x_83, 1, x_81); -lean_ctor_set(x_83, 2, x_80); -lean_ctor_set(x_83, 3, x_76); -lean_ctor_set_uint8(x_83, sizeof(void*)*4, x_82); -x_84 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_84, 0, x_83); -x_85 = l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_expandDeclId___spec__11(x_84, x_2, x_3, x_77); -x_86 = lean_ctor_get(x_85, 1); -lean_inc(x_86); -if (lean_is_exclusive(x_85)) { - lean_ctor_release(x_85, 0); - lean_ctor_release(x_85, 1); - x_87 = x_85; -} else { - lean_dec_ref(x_85); - x_87 = lean_box(0); -} -lean_inc(x_1); -x_88 = lean_private_to_user_name(x_1); -if (lean_obj_tag(x_88) == 0) -{ -lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; -x_89 = l_Lean_MessageData_ofName(x_1); -x_90 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__8; -if (lean_is_scalar(x_87)) { - x_91 = lean_alloc_ctor(7, 2, 0); -} else { - x_91 = x_87; - lean_ctor_set_tag(x_91, 7); -} -lean_ctor_set(x_91, 0, x_90); -lean_ctor_set(x_91, 1, x_89); -x_92 = l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_addUnivLevel___spec__1___closed__4; -lean_ctor_set_tag(x_5, 7); -lean_ctor_set(x_5, 1, x_92); -lean_ctor_set(x_5, 0, x_91); -x_93 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_5, x_2, x_3, x_86); -x_94 = lean_ctor_get(x_93, 0); -lean_inc(x_94); -x_95 = lean_ctor_get(x_93, 1); -lean_inc(x_95); -if (lean_is_exclusive(x_93)) { - lean_ctor_release(x_93, 0); - lean_ctor_release(x_93, 1); - x_96 = x_93; -} else { - lean_dec_ref(x_93); - x_96 = lean_box(0); -} -if (lean_is_scalar(x_96)) { - x_97 = lean_alloc_ctor(1, 2, 0); -} else { - x_97 = x_96; -} -lean_ctor_set(x_97, 0, x_94); -lean_ctor_set(x_97, 1, x_95); -return x_97; -} -else -{ -lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; -lean_dec(x_1); -x_98 = lean_ctor_get(x_88, 0); -lean_inc(x_98); -lean_dec(x_88); -x_99 = l_Lean_MessageData_ofName(x_98); -x_100 = l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___closed__2; -if (lean_is_scalar(x_87)) { - x_101 = lean_alloc_ctor(7, 2, 0); -} else { - x_101 = x_87; - lean_ctor_set_tag(x_101, 7); -} -lean_ctor_set(x_101, 0, x_100); -lean_ctor_set(x_101, 1, x_99); -x_102 = l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_addUnivLevel___spec__1___closed__4; -lean_ctor_set_tag(x_5, 7); -lean_ctor_set(x_5, 1, x_102); -lean_ctor_set(x_5, 0, x_101); -x_103 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_5, x_2, x_3, x_86); -x_104 = lean_ctor_get(x_103, 0); -lean_inc(x_104); -x_105 = lean_ctor_get(x_103, 1); -lean_inc(x_105); -if (lean_is_exclusive(x_103)) { - lean_ctor_release(x_103, 0); - lean_ctor_release(x_103, 1); - 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(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; -} -} -else -{ -lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; -lean_dec(x_73); -lean_free_object(x_5); -lean_dec(x_2); -lean_dec(x_1); -x_108 = lean_ctor_get(x_75, 0); -lean_inc(x_108); -x_109 = lean_ctor_get(x_75, 1); -lean_inc(x_109); -if (lean_is_exclusive(x_75)) { - lean_ctor_release(x_75, 0); - lean_ctor_release(x_75, 1); - x_110 = x_75; -} else { - lean_dec_ref(x_75); - x_110 = lean_box(0); -} -if (lean_is_scalar(x_110)) { - x_111 = lean_alloc_ctor(1, 2, 0); -} else { - x_111 = x_110; -} -lean_ctor_set(x_111, 0, x_108); -lean_ctor_set(x_111, 1, x_109); -return x_111; -} -} -} -} -else -{ -lean_object* x_112; lean_object* x_113; lean_object* x_114; uint8_t x_115; -x_112 = lean_ctor_get(x_5, 0); -x_113 = lean_ctor_get(x_5, 1); -lean_inc(x_113); -lean_inc(x_112); -lean_dec(x_5); -x_114 = lean_ctor_get(x_112, 0); -lean_inc(x_114); -lean_dec(x_112); -lean_inc(x_114); -x_115 = l_Lean_Environment_contains(x_114, x_1); -if (x_115 == 0) -{ -lean_object* x_116; lean_object* x_117; -x_116 = lean_box(0); -x_117 = l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__3(x_1, x_114, x_116, x_2, x_3, x_113); -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_dec(x_114); -x_118 = l_Lean_Elab_Command_getRef(x_2, x_3, x_113); -x_119 = lean_ctor_get(x_118, 0); -lean_inc(x_119); -x_120 = lean_ctor_get(x_118, 1); -lean_inc(x_120); -if (lean_is_exclusive(x_118)) { - lean_ctor_release(x_118, 0); - lean_ctor_release(x_118, 1); - x_121 = x_118; -} else { - lean_dec_ref(x_118); - x_121 = lean_box(0); -} -lean_inc(x_2); -lean_inc(x_1); -x_122 = l_Lean_mkConstWithLevelParams___at_Lean_Elab_Command_expandDeclId___spec__8(x_1, x_2, x_3, 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; lean_object* x_127; lean_object* x_128; uint8_t x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; -x_123 = lean_ctor_get(x_122, 0); -lean_inc(x_123); -x_124 = lean_ctor_get(x_122, 1); -lean_inc(x_124); -lean_dec(x_122); -x_125 = lean_box(0); -if (lean_is_scalar(x_121)) { - x_126 = lean_alloc_ctor(0, 2, 0); -} else { - x_126 = x_121; -} -lean_ctor_set(x_126, 0, x_125); -lean_ctor_set(x_126, 1, x_119); -x_127 = lean_box(0); -x_128 = l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1___closed__2; -x_129 = 0; -x_130 = lean_alloc_ctor(0, 4, 1); -lean_ctor_set(x_130, 0, x_126); -lean_ctor_set(x_130, 1, x_128); -lean_ctor_set(x_130, 2, x_127); -lean_ctor_set(x_130, 3, x_123); -lean_ctor_set_uint8(x_130, sizeof(void*)*4, x_129); -x_131 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_131, 0, x_130); -x_132 = l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_expandDeclId___spec__11(x_131, x_2, x_3, x_124); -x_133 = lean_ctor_get(x_132, 1); -lean_inc(x_133); -if (lean_is_exclusive(x_132)) { - lean_ctor_release(x_132, 0); - lean_ctor_release(x_132, 1); - x_134 = x_132; -} else { - lean_dec_ref(x_132); - x_134 = lean_box(0); -} -lean_inc(x_1); -x_135 = lean_private_to_user_name(x_1); -if (lean_obj_tag(x_135) == 0) -{ -lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; -x_136 = l_Lean_MessageData_ofName(x_1); -x_137 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__8; -if (lean_is_scalar(x_134)) { - x_138 = lean_alloc_ctor(7, 2, 0); -} else { - x_138 = x_134; - lean_ctor_set_tag(x_138, 7); -} -lean_ctor_set(x_138, 0, x_137); -lean_ctor_set(x_138, 1, x_136); -x_139 = l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_addUnivLevel___spec__1___closed__4; -x_140 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_140, 0, x_138); -lean_ctor_set(x_140, 1, x_139); -x_141 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_140, x_2, x_3, x_133); -x_142 = lean_ctor_get(x_141, 0); -lean_inc(x_142); -x_143 = lean_ctor_get(x_141, 1); -lean_inc(x_143); -if (lean_is_exclusive(x_141)) { - lean_ctor_release(x_141, 0); - lean_ctor_release(x_141, 1); - x_144 = x_141; -} else { - lean_dec_ref(x_141); - x_144 = lean_box(0); -} -if (lean_is_scalar(x_144)) { - x_145 = lean_alloc_ctor(1, 2, 0); -} else { - x_145 = x_144; -} -lean_ctor_set(x_145, 0, x_142); -lean_ctor_set(x_145, 1, x_143); -return x_145; -} -else -{ -lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_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_dec(x_1); -x_146 = lean_ctor_get(x_135, 0); -lean_inc(x_146); -lean_dec(x_135); -x_147 = l_Lean_MessageData_ofName(x_146); -x_148 = l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___closed__2; -if (lean_is_scalar(x_134)) { - x_149 = lean_alloc_ctor(7, 2, 0); -} else { - x_149 = x_134; - lean_ctor_set_tag(x_149, 7); -} -lean_ctor_set(x_149, 0, x_148); -lean_ctor_set(x_149, 1, x_147); -x_150 = l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_addUnivLevel___spec__1___closed__4; -x_151 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_151, 0, x_149); -lean_ctor_set(x_151, 1, x_150); -x_152 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_151, x_2, x_3, x_133); -x_153 = lean_ctor_get(x_152, 0); -lean_inc(x_153); -x_154 = lean_ctor_get(x_152, 1); -lean_inc(x_154); -if (lean_is_exclusive(x_152)) { - lean_ctor_release(x_152, 0); - lean_ctor_release(x_152, 1); - x_155 = x_152; -} else { - lean_dec_ref(x_152); - x_155 = lean_box(0); -} -if (lean_is_scalar(x_155)) { - x_156 = lean_alloc_ctor(1, 2, 0); -} else { - x_156 = x_155; -} -lean_ctor_set(x_156, 0, x_153); -lean_ctor_set(x_156, 1, x_154); -return x_156; -} -} -else -{ -lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; -lean_dec(x_121); -lean_dec(x_119); -lean_dec(x_2); -lean_dec(x_1); -x_157 = lean_ctor_get(x_122, 0); -lean_inc(x_157); -x_158 = lean_ctor_get(x_122, 1); -lean_inc(x_158); -if (lean_is_exclusive(x_122)) { - lean_ctor_release(x_122, 0); - lean_ctor_release(x_122, 1); - x_159 = x_122; -} else { - lean_dec_ref(x_122); - x_159 = lean_box(0); -} -if (lean_is_scalar(x_159)) { - x_160 = lean_alloc_ctor(1, 2, 0); -} else { - x_160 = x_159; -} -lean_ctor_set(x_160, 0, x_157); -lean_ctor_set(x_160, 1, x_158); -return x_160; -} -} -} -} -} -static lean_object* _init_l_Lean_Elab_applyVisibility___at_Lean_Elab_Command_expandDeclId___spec__6___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_protectedExt; -return x_1; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_applyVisibility___at_Lean_Elab_Command_expandDeclId___spec__6(uint8_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -switch (x_1) { -case 0: -{ -lean_object* x_6; -lean_inc(x_2); -x_6 = l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7(x_2, x_3, x_4, x_5); -if (lean_obj_tag(x_6) == 0) -{ -uint8_t x_7; -x_7 = !lean_is_exclusive(x_6); -if (x_7 == 0) -{ -lean_object* x_8; -x_8 = lean_ctor_get(x_6, 0); -lean_dec(x_8); -lean_ctor_set(x_6, 0, x_2); -return x_6; -} -else -{ -lean_object* x_9; lean_object* x_10; -x_9 = lean_ctor_get(x_6, 1); -lean_inc(x_9); -lean_dec(x_6); -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_2); -lean_ctor_set(x_10, 1, x_9); -return x_10; -} -} -else -{ -uint8_t x_11; -lean_dec(x_2); -x_11 = !lean_is_exclusive(x_6); -if (x_11 == 0) -{ -return x_6; -} -else -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_12 = lean_ctor_get(x_6, 0); -x_13 = lean_ctor_get(x_6, 1); -lean_inc(x_13); -lean_inc(x_12); -lean_dec(x_6); -x_14 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_14, 0, x_12); -lean_ctor_set(x_14, 1, x_13); -return x_14; -} -} -} -case 1: -{ -lean_object* x_15; -lean_inc(x_2); -x_15 = l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7(x_2, x_3, x_4, x_5); -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; -x_16 = lean_ctor_get(x_15, 1); -lean_inc(x_16); -lean_dec(x_15); -x_17 = lean_st_ref_take(x_4, x_16); -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_17, 1); -lean_inc(x_19); -lean_dec(x_17); -x_20 = !lean_is_exclusive(x_18); -if (x_20 == 0) -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; -x_21 = lean_ctor_get(x_18, 0); -x_22 = l_Lean_Elab_applyVisibility___at_Lean_Elab_Command_expandDeclId___spec__6___closed__1; -lean_inc(x_2); -x_23 = l_Lean_TagDeclarationExtension_tag(x_22, x_21, x_2); -lean_ctor_set(x_18, 0, x_23); -x_24 = lean_st_ref_set(x_4, x_18, x_19); -x_25 = !lean_is_exclusive(x_24); -if (x_25 == 0) -{ -lean_object* x_26; -x_26 = lean_ctor_get(x_24, 0); -lean_dec(x_26); -lean_ctor_set(x_24, 0, x_2); -return x_24; -} -else -{ -lean_object* x_27; lean_object* x_28; -x_27 = lean_ctor_get(x_24, 1); -lean_inc(x_27); -lean_dec(x_24); -x_28 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_28, 0, x_2); -lean_ctor_set(x_28, 1, x_27); -return x_28; -} -} -else -{ -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; 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_18, 0); -x_30 = lean_ctor_get(x_18, 1); -x_31 = lean_ctor_get(x_18, 2); -x_32 = lean_ctor_get(x_18, 3); -x_33 = lean_ctor_get(x_18, 4); -x_34 = lean_ctor_get(x_18, 5); -x_35 = lean_ctor_get(x_18, 6); -x_36 = lean_ctor_get(x_18, 7); -lean_inc(x_36); -lean_inc(x_35); -lean_inc(x_34); -lean_inc(x_33); -lean_inc(x_32); -lean_inc(x_31); -lean_inc(x_30); -lean_inc(x_29); -lean_dec(x_18); -x_37 = l_Lean_Elab_applyVisibility___at_Lean_Elab_Command_expandDeclId___spec__6___closed__1; -lean_inc(x_2); -x_38 = l_Lean_TagDeclarationExtension_tag(x_37, x_29, x_2); -x_39 = lean_alloc_ctor(0, 8, 0); -lean_ctor_set(x_39, 0, x_38); -lean_ctor_set(x_39, 1, x_30); -lean_ctor_set(x_39, 2, x_31); -lean_ctor_set(x_39, 3, x_32); -lean_ctor_set(x_39, 4, x_33); -lean_ctor_set(x_39, 5, x_34); -lean_ctor_set(x_39, 6, x_35); -lean_ctor_set(x_39, 7, x_36); -x_40 = lean_st_ref_set(x_4, x_39, x_19); -x_41 = lean_ctor_get(x_40, 1); -lean_inc(x_41); -if (lean_is_exclusive(x_40)) { - lean_ctor_release(x_40, 0); - lean_ctor_release(x_40, 1); - x_42 = x_40; -} else { - lean_dec_ref(x_40); - x_42 = lean_box(0); -} -if (lean_is_scalar(x_42)) { - x_43 = lean_alloc_ctor(0, 2, 0); -} else { - x_43 = x_42; -} -lean_ctor_set(x_43, 0, x_2); -lean_ctor_set(x_43, 1, x_41); -return x_43; -} -} -else -{ -uint8_t x_44; -lean_dec(x_2); -x_44 = !lean_is_exclusive(x_15); -if (x_44 == 0) -{ -return x_15; -} -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_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; -} -} -} -default: -{ -lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; -x_48 = lean_st_ref_get(x_4, x_5); -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_52 = l_Lean_mkPrivateName(x_51, x_2); -lean_inc(x_52); -x_53 = l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7(x_52, x_3, x_4, x_50); -if (lean_obj_tag(x_53) == 0) -{ -uint8_t x_54; -x_54 = !lean_is_exclusive(x_53); -if (x_54 == 0) -{ -lean_object* x_55; -x_55 = lean_ctor_get(x_53, 0); -lean_dec(x_55); -lean_ctor_set(x_53, 0, x_52); -return x_53; -} -else -{ -lean_object* x_56; lean_object* x_57; -x_56 = lean_ctor_get(x_53, 1); -lean_inc(x_56); -lean_dec(x_53); -x_57 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_57, 0, x_52); -lean_ctor_set(x_57, 1, x_56); -return x_57; -} -} -else -{ -uint8_t x_58; -lean_dec(x_52); -x_58 = !lean_is_exclusive(x_53); -if (x_58 == 0) -{ -return x_53; -} -else -{ -lean_object* x_59; lean_object* x_60; lean_object* x_61; -x_59 = lean_ctor_get(x_53, 0); -x_60 = lean_ctor_get(x_53, 1); -lean_inc(x_60); -lean_inc(x_59); -lean_dec(x_53); -x_61 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_61, 0, x_59); -lean_ctor_set(x_61, 1, x_60); -return x_61; -} -} -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___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; lean_object* x_8; -x_7 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_7, 0, x_1); -lean_ctor_set(x_7, 1, x_2); -x_8 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_8, 0, x_7); -lean_ctor_set(x_8, 1, x_6); -return x_8; -} -} -static lean_object* _init_l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___lambda__2___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("protected declarations must be in a namespace", 45, 45); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___lambda__2___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___lambda__2___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; -lean_inc(x_6); -lean_inc(x_1); -x_9 = l_Lean_Elab_checkIfShadowingStructureField___at_Lean_Elab_Command_expandDeclId___spec__3(x_1, 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 = lean_ctor_get_uint8(x_2, sizeof(void*)*2); -lean_inc(x_6); -x_12 = l_Lean_Elab_applyVisibility___at_Lean_Elab_Command_expandDeclId___spec__6(x_11, x_1, x_6, x_7, x_10); -if (lean_obj_tag(x_12) == 0) -{ -lean_object* x_13; -x_13 = lean_box(x_11); -if (lean_obj_tag(x_13) == 1) -{ -if (lean_obj_tag(x_3) == 1) -{ -uint8_t x_14; -lean_dec(x_6); -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, 0); -x_16 = lean_ctor_get(x_3, 1); -lean_inc(x_16); -lean_dec(x_3); -x_17 = lean_box(0); -x_18 = l_Lean_Name_str___override(x_17, x_16); -x_19 = l_Lean_Name_append(x_18, x_4); -x_20 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_20, 0, x_15); -lean_ctor_set(x_20, 1, x_19); -lean_ctor_set(x_12, 0, x_20); -return x_12; -} -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; -x_21 = lean_ctor_get(x_12, 0); -x_22 = lean_ctor_get(x_12, 1); -lean_inc(x_22); -lean_inc(x_21); -lean_dec(x_12); -x_23 = lean_ctor_get(x_3, 1); -lean_inc(x_23); -lean_dec(x_3); -x_24 = lean_box(0); -x_25 = l_Lean_Name_str___override(x_24, x_23); -x_26 = l_Lean_Name_append(x_25, x_4); -x_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_21); -lean_ctor_set(x_27, 1, x_26); -x_28 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_28, 0, x_27); -lean_ctor_set(x_28, 1, x_22); -return x_28; -} -} -else -{ -lean_object* x_29; lean_object* x_30; uint8_t x_31; -lean_dec(x_3); -x_29 = lean_ctor_get(x_12, 0); -lean_inc(x_29); -x_30 = lean_ctor_get(x_12, 1); -lean_inc(x_30); -lean_dec(x_12); -x_31 = l_Lean_Name_isAtomic(x_4); -if (x_31 == 0) -{ -lean_object* x_32; lean_object* x_33; -x_32 = lean_box(0); -x_33 = l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___lambda__1(x_29, x_4, x_32, x_6, x_7, x_30); -lean_dec(x_6); -return x_33; -} -else -{ -lean_object* x_34; lean_object* x_35; uint8_t x_36; -lean_dec(x_29); -lean_dec(x_4); -x_34 = l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___lambda__2___closed__2; -x_35 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_34, x_6, x_7, x_30); -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; -} -} -} -} -else -{ -uint8_t x_40; -lean_dec(x_13); -lean_dec(x_6); -lean_dec(x_3); -x_40 = !lean_is_exclusive(x_12); -if (x_40 == 0) -{ -lean_object* x_41; lean_object* x_42; -x_41 = lean_ctor_get(x_12, 0); -x_42 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_42, 0, x_41); -lean_ctor_set(x_42, 1, x_4); -lean_ctor_set(x_12, 0, x_42); -return x_12; -} -else -{ -lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_43 = lean_ctor_get(x_12, 0); -x_44 = lean_ctor_get(x_12, 1); -lean_inc(x_44); -lean_inc(x_43); -lean_dec(x_12); -x_45 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_45, 0, x_43); -lean_ctor_set(x_45, 1, x_4); -x_46 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_46, 0, x_45); -lean_ctor_set(x_46, 1, x_44); -return x_46; -} -} -} -else -{ -uint8_t x_47; -lean_dec(x_6); -lean_dec(x_4); -lean_dec(x_3); -x_47 = !lean_is_exclusive(x_12); -if (x_47 == 0) -{ -return x_12; -} -else -{ -lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_ctor_get(x_12, 0); -x_49 = lean_ctor_get(x_12, 1); -lean_inc(x_49); -lean_inc(x_48); -lean_dec(x_12); -x_50 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_50, 0, x_48); -lean_ctor_set(x_50, 1, x_49); -return x_50; -} -} -} -else -{ -uint8_t x_51; -lean_dec(x_6); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_51 = !lean_is_exclusive(x_9); -if (x_51 == 0) -{ -return x_9; -} -else -{ -lean_object* x_52; lean_object* x_53; lean_object* x_54; -x_52 = lean_ctor_get(x_9, 0); -x_53 = lean_ctor_get(x_9, 1); -lean_inc(x_53); -lean_inc(x_52); -lean_dec(x_9); -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_EXPORT lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -uint8_t x_12; -if (x_5 == 0) -{ -uint8_t x_43; -x_43 = 0; -x_12 = x_43; -goto block_42; -} -else -{ -uint8_t x_44; -x_44 = 1; -x_12 = x_44; -goto block_42; -} -block_42: -{ -lean_object* x_13; -if (x_12 == 0) -{ -lean_object* x_34; -lean_inc(x_7); -lean_inc(x_6); -x_34 = l_Lean_Name_append(x_6, x_7); -x_13 = x_34; -goto block_33; -} -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; -x_35 = lean_box(0); -lean_inc(x_2); -x_36 = l_Lean_Name_replacePrefix(x_2, x_3, x_35); -x_37 = lean_ctor_get(x_4, 1); -x_38 = lean_ctor_get(x_4, 2); -x_39 = lean_ctor_get(x_4, 3); -lean_inc(x_39); -lean_inc(x_38); -lean_inc(x_37); -x_40 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_40, 0, x_36); -lean_ctor_set(x_40, 1, x_37); -lean_ctor_set(x_40, 2, x_38); -lean_ctor_set(x_40, 3, x_39); -x_41 = l_Lean_MacroScopesView_review(x_40); -x_13 = x_41; -goto block_33; -} -block_33: -{ -if (x_12 == 0) -{ -lean_object* x_14; lean_object* x_15; -lean_dec(x_2); -x_14 = lean_box(0); -x_15 = l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___lambda__2(x_13, x_1, x_6, x_7, x_14, x_9, x_10, x_11); -return x_15; -} -else -{ -lean_dec(x_7); -lean_dec(x_6); -if (lean_obj_tag(x_2) == 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_object* x_22; -x_16 = lean_ctor_get(x_2, 0); -lean_inc(x_16); -x_17 = lean_ctor_get(x_2, 1); -lean_inc(x_17); -lean_dec(x_2); -x_18 = lean_box(0); -x_19 = l_Lean_Name_str___override(x_18, x_17); -x_20 = l_Lean_Name_replacePrefix(x_16, x_3, x_18); -x_21 = lean_box(0); -x_22 = l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___lambda__2(x_13, x_1, x_20, x_19, x_21, x_9, x_10, x_11); -return x_22; -} -else -{ -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; -lean_dec(x_13); -x_23 = l_Lean_MessageData_ofName(x_2); -x_24 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__2; -x_25 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_25, 0, x_24); -lean_ctor_set(x_25, 1, x_23); -x_26 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__8; -x_27 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_26); -x_28 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_27, x_9, x_10, x_11); -x_29 = !lean_is_exclusive(x_28); -if (x_29 == 0) -{ -return x_28; -} -else -{ -lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_30 = lean_ctor_get(x_28, 0); -x_31 = lean_ctor_get(x_28, 1); -lean_inc(x_31); -lean_inc(x_30); -lean_dec(x_28); -x_32 = lean_alloc_ctor(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_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("_root_", 6, 6); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("invalid declaration name `_root_`, `_root_` is a prefix used to refer to the 'root' namespace", 93, 93); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___closed__3; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; uint8_t x_11; -lean_inc(x_3); -x_7 = l_Lean_extractMacroScopes(x_3); -x_8 = lean_ctor_get(x_7, 0); -lean_inc(x_8); -x_9 = l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___closed__2; -x_10 = l_Lean_Name_isPrefixOf(x_9, x_8); -x_11 = lean_name_eq(x_8, x_9); -if (x_11 == 0) -{ -lean_object* x_12; lean_object* x_13; -x_12 = lean_box(0); -x_13 = l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___lambda__3(x_2, x_8, x_9, x_7, x_10, x_1, x_3, x_12, x_4, x_5, x_6); -lean_dec(x_7); -return x_13; -} -else -{ -lean_object* x_14; lean_object* x_15; uint8_t x_16; -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_1); -x_14 = l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___closed__4; -x_15 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_14, x_4, x_5, x_6); -x_16 = !lean_is_exclusive(x_15); -if (x_16 == 0) -{ -return x_15; -} -else -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_15, 0); -x_18 = lean_ctor_get(x_15, 1); -lean_inc(x_18); -lean_inc(x_17); -lean_dec(x_15); -x_19 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_19, 0, x_17); -lean_ctor_set(x_19, 1, x_18); -return x_19; -} -} -} -} -static lean_object* _init_l_Lean_addDocString___at_Lean_Elab_Command_expandDeclId___spec__14___lambda__1___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_docStringExt; -return x_1; -} -} -LEAN_EXPORT lean_object* l_Lean_addDocString___at_Lean_Elab_Command_expandDeclId___spec__14___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; lean_object* x_9; uint8_t x_10; -x_7 = lean_st_ref_take(x_5, x_6); -x_8 = lean_ctor_get(x_7, 0); -lean_inc(x_8); -x_9 = lean_ctor_get(x_7, 1); -lean_inc(x_9); -lean_dec(x_7); -x_10 = !lean_is_exclusive(x_8); -if (x_10 == 0) -{ -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; -x_11 = lean_ctor_get(x_8, 0); -x_12 = l_String_removeLeadingSpaces(x_1); -x_13 = l_Lean_addDocString___at_Lean_Elab_Command_expandDeclId___spec__14___lambda__1___closed__1; -x_14 = l_Lean_MapDeclarationExtension_insert___rarg(x_13, x_11, x_2, x_12); -lean_ctor_set(x_8, 0, x_14); -x_15 = lean_st_ref_set(x_5, x_8, x_9); -x_16 = !lean_is_exclusive(x_15); -if (x_16 == 0) -{ -lean_object* x_17; lean_object* x_18; -x_17 = lean_ctor_get(x_15, 0); -lean_dec(x_17); -x_18 = lean_box(0); -lean_ctor_set(x_15, 0, x_18); -return x_15; -} -else -{ -lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_19 = lean_ctor_get(x_15, 1); -lean_inc(x_19); -lean_dec(x_15); -x_20 = lean_box(0); -x_21 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_21, 0, x_20); -lean_ctor_set(x_21, 1, x_19); -return x_21; -} -} -else -{ -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_22 = lean_ctor_get(x_8, 0); -x_23 = lean_ctor_get(x_8, 1); -x_24 = lean_ctor_get(x_8, 2); -x_25 = lean_ctor_get(x_8, 3); -x_26 = lean_ctor_get(x_8, 4); -x_27 = lean_ctor_get(x_8, 5); -x_28 = lean_ctor_get(x_8, 6); -x_29 = lean_ctor_get(x_8, 7); -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_dec(x_8); -x_30 = l_String_removeLeadingSpaces(x_1); -x_31 = l_Lean_addDocString___at_Lean_Elab_Command_expandDeclId___spec__14___lambda__1___closed__1; -x_32 = l_Lean_MapDeclarationExtension_insert___rarg(x_31, x_22, x_2, x_30); -x_33 = lean_alloc_ctor(0, 8, 0); -lean_ctor_set(x_33, 0, x_32); -lean_ctor_set(x_33, 1, x_23); -lean_ctor_set(x_33, 2, x_24); -lean_ctor_set(x_33, 3, x_25); -lean_ctor_set(x_33, 4, x_26); -lean_ctor_set(x_33, 5, x_27); -lean_ctor_set(x_33, 6, x_28); -lean_ctor_set(x_33, 7, x_29); -x_34 = lean_st_ref_set(x_5, x_33, x_9); -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); -} -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; -} -} -} -static lean_object* _init_l_Lean_addDocString___at_Lean_Elab_Command_expandDeclId___spec__14___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("invalid doc string, declaration '", 33, 33); -return x_1; -} -} -static lean_object* _init_l_Lean_addDocString___at_Lean_Elab_Command_expandDeclId___spec__14___closed__2() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("' is in an imported module", 26, 26); -return x_1; -} -} -LEAN_EXPORT lean_object* l_Lean_addDocString___at_Lean_Elab_Command_expandDeclId___spec__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; -x_6 = lean_st_ref_get(x_4, x_5); -x_7 = lean_ctor_get(x_6, 0); -lean_inc(x_7); -x_8 = lean_ctor_get(x_6, 1); -lean_inc(x_8); -lean_dec(x_6); -x_9 = lean_ctor_get(x_7, 0); -lean_inc(x_9); -lean_dec(x_7); -x_10 = l_Lean_Environment_getModuleIdxFor_x3f(x_9, x_1); -lean_dec(x_9); -if (lean_obj_tag(x_10) == 0) -{ -lean_object* x_11; lean_object* x_12; -x_11 = lean_box(0); -x_12 = l_Lean_addDocString___at_Lean_Elab_Command_expandDeclId___spec__14___lambda__1(x_2, x_1, x_11, x_3, x_4, x_8); -lean_dec(x_3); -return x_12; -} -else -{ -uint8_t x_13; -lean_dec(x_2); -x_13 = !lean_is_exclusive(x_10); -if (x_13 == 0) -{ -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; uint8_t x_24; -x_14 = lean_ctor_get(x_10, 0); -lean_dec(x_14); -x_15 = 1; -x_16 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_runLinters___spec__9___closed__1; -x_17 = l_Lean_Name_toString(x_1, x_15, x_16); -x_18 = l_Lean_addDocString___at_Lean_Elab_Command_expandDeclId___spec__14___closed__1; -x_19 = lean_string_append(x_18, x_17); -lean_dec(x_17); -x_20 = l_Lean_addDocString___at_Lean_Elab_Command_expandDeclId___spec__14___closed__2; -x_21 = lean_string_append(x_19, x_20); -lean_ctor_set_tag(x_10, 3); -lean_ctor_set(x_10, 0, x_21); -x_22 = l_Lean_MessageData_ofFormat(x_10); -x_23 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_22, x_3, x_4, x_8); -x_24 = !lean_is_exclusive(x_23); -if (x_24 == 0) -{ -return x_23; -} -else -{ -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_23, 0); -x_26 = lean_ctor_get(x_23, 1); -lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_23); -x_27 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_26); -return x_27; -} -} -else -{ -uint8_t x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; -lean_dec(x_10); -x_28 = 1; -x_29 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_runLinters___spec__9___closed__1; -x_30 = l_Lean_Name_toString(x_1, x_28, x_29); -x_31 = l_Lean_addDocString___at_Lean_Elab_Command_expandDeclId___spec__14___closed__1; -x_32 = lean_string_append(x_31, x_30); -lean_dec(x_30); -x_33 = l_Lean_addDocString___at_Lean_Elab_Command_expandDeclId___spec__14___closed__2; -x_34 = lean_string_append(x_32, x_33); -x_35 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_35, 0, x_34); -x_36 = l_Lean_MessageData_ofFormat(x_35); -x_37 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_36, x_3, x_4, x_8); -x_38 = lean_ctor_get(x_37, 0); -lean_inc(x_38); -x_39 = lean_ctor_get(x_37, 1); -lean_inc(x_39); -if (lean_is_exclusive(x_37)) { - lean_ctor_release(x_37, 0); - lean_ctor_release(x_37, 1); - x_40 = x_37; -} else { - lean_dec_ref(x_37); - x_40 = lean_box(0); -} -if (lean_is_scalar(x_40)) { - x_41 = lean_alloc_ctor(1, 2, 0); -} else { - x_41 = x_40; -} -lean_ctor_set(x_41, 0, x_38); -lean_ctor_set(x_41, 1, x_39); -return x_41; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_addDocString_x27___at_Lean_Elab_Command_expandDeclId___spec__13(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -if (lean_obj_tag(x_2) == 0) -{ -lean_object* x_6; lean_object* x_7; -lean_dec(x_3); -lean_dec(x_1); -x_6 = lean_box(0); -x_7 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_7, 0, x_6); -lean_ctor_set(x_7, 1, x_5); -return x_7; -} -else -{ -lean_object* x_8; lean_object* x_9; -x_8 = lean_ctor_get(x_2, 0); -lean_inc(x_8); -lean_dec(x_2); -x_9 = l_Lean_addDocString___at_Lean_Elab_Command_expandDeclId___spec__14(x_1, x_8, x_3, x_4, x_5); -return x_9; -} -} -} -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___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; uint8_t x_11; -x_5 = l_Lean_Elab_Command_getRef(x_2, x_3, x_4); -x_6 = lean_ctor_get(x_5, 0); -lean_inc(x_6); -x_7 = lean_ctor_get(x_5, 1); -lean_inc(x_7); -lean_dec(x_5); -x_8 = lean_ctor_get(x_2, 4); -lean_inc(x_8); -lean_inc(x_8); -x_9 = l_Lean_Elab_getBetterRef(x_6, x_8); -lean_dec(x_6); -x_10 = l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1(x_1, x_2, x_3, x_7); -x_11 = !lean_is_exclusive(x_10); -if (x_11 == 0) -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; -x_12 = lean_ctor_get(x_10, 0); -x_13 = lean_ctor_get(x_10, 1); -x_14 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_12, x_8, x_2, x_3, x_13); -lean_dec(x_2); -x_15 = !lean_is_exclusive(x_14); -if (x_15 == 0) -{ -lean_object* x_16; -x_16 = lean_ctor_get(x_14, 0); -lean_ctor_set(x_10, 1, x_16); -lean_ctor_set(x_10, 0, x_9); -lean_ctor_set_tag(x_14, 1); -lean_ctor_set(x_14, 0, x_10); -return x_14; -} -else -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_14, 0); -x_18 = lean_ctor_get(x_14, 1); -lean_inc(x_18); -lean_inc(x_17); -lean_dec(x_14); -lean_ctor_set(x_10, 1, x_17); -lean_ctor_set(x_10, 0, x_9); -x_19 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_19, 0, x_10); -lean_ctor_set(x_19, 1, 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; lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_20 = lean_ctor_get(x_10, 0); -x_21 = lean_ctor_get(x_10, 1); -lean_inc(x_21); -lean_inc(x_20); -lean_dec(x_10); -x_22 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_20, x_8, x_2, x_3, x_21); -lean_dec(x_2); -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -x_24 = lean_ctor_get(x_22, 1); -lean_inc(x_24); -if (lean_is_exclusive(x_22)) { - lean_ctor_release(x_22, 0); - lean_ctor_release(x_22, 1); - x_25 = x_22; -} else { - lean_dec_ref(x_22); - x_25 = lean_box(0); -} -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_9); -lean_ctor_set(x_26, 1, x_23); -if (lean_is_scalar(x_25)) { - x_27 = lean_alloc_ctor(1, 2, 0); -} else { - x_27 = x_25; - lean_ctor_set_tag(x_27, 1); -} -lean_ctor_set(x_27, 0, x_26); -lean_ctor_set(x_27, 1, x_24); -return x_27; -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_expandDeclId___spec__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; -x_5 = l_Lean_MessageData_ofName(x_1); -x_6 = l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_addUnivLevel___spec__1___closed__2; -x_7 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_7, 0, x_6); -lean_ctor_set(x_7, 1, x_5); -x_8 = l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_addUnivLevel___spec__1___closed__4; -x_9 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_9, 0, x_7); -lean_ctor_set(x_9, 1, x_8); -x_10 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__16(x_9, x_2, x_3, x_4); -return x_10; -} -} -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_expandDeclId___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) { -_start: -{ -uint8_t x_8; -x_8 = lean_usize_dec_eq(x_2, x_3); -if (x_8 == 0) -{ -lean_object* x_9; lean_object* x_10; uint8_t x_11; -x_9 = lean_array_uget(x_1, x_2); -x_10 = l_Lean_Syntax_getId(x_9); -x_11 = l_List_elem___at_Lean_addAliasEntry___spec__16(x_10, x_4); -if (x_11 == 0) -{ -lean_object* x_12; size_t x_13; size_t x_14; -lean_dec(x_9); -x_12 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_12, 0, x_10); -lean_ctor_set(x_12, 1, x_4); -x_13 = 1; -x_14 = lean_usize_add(x_2, x_13); -x_2 = x_14; -x_4 = x_12; -goto _start; -} -else -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; -lean_dec(x_4); -x_16 = l_Lean_Elab_Command_getRef(x_5, x_6, x_7); -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_replaceRef(x_9, x_17); -lean_dec(x_17); -lean_dec(x_9); -x_20 = !lean_is_exclusive(x_5); -if (x_20 == 0) -{ -lean_object* x_21; lean_object* x_22; uint8_t x_23; -x_21 = lean_ctor_get(x_5, 6); -lean_dec(x_21); -lean_ctor_set(x_5, 6, x_19); -x_22 = l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_expandDeclId___spec__15(x_10, x_5, x_6, x_18); -x_23 = !lean_is_exclusive(x_22); -if (x_23 == 0) -{ -return x_22; -} -else -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_22, 0); -x_25 = lean_ctor_get(x_22, 1); -lean_inc(x_25); -lean_inc(x_24); -lean_dec(x_22); -x_26 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_26, 0, x_24); -lean_ctor_set(x_26, 1, x_25); -return x_26; -} -} -else -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_27 = lean_ctor_get(x_5, 0); -x_28 = lean_ctor_get(x_5, 1); -x_29 = lean_ctor_get(x_5, 2); -x_30 = lean_ctor_get(x_5, 3); -x_31 = lean_ctor_get(x_5, 4); -x_32 = lean_ctor_get(x_5, 5); -x_33 = lean_ctor_get(x_5, 7); -x_34 = lean_ctor_get(x_5, 8); -x_35 = lean_ctor_get(x_5, 9); -x_36 = lean_ctor_get_uint8(x_5, sizeof(void*)*10); -lean_inc(x_35); -lean_inc(x_34); -lean_inc(x_33); -lean_inc(x_32); -lean_inc(x_31); -lean_inc(x_30); -lean_inc(x_29); -lean_inc(x_28); -lean_inc(x_27); -lean_dec(x_5); -x_37 = lean_alloc_ctor(0, 10, 1); -lean_ctor_set(x_37, 0, x_27); -lean_ctor_set(x_37, 1, x_28); -lean_ctor_set(x_37, 2, x_29); -lean_ctor_set(x_37, 3, x_30); -lean_ctor_set(x_37, 4, x_31); -lean_ctor_set(x_37, 5, x_32); -lean_ctor_set(x_37, 6, x_19); -lean_ctor_set(x_37, 7, x_33); -lean_ctor_set(x_37, 8, x_34); -lean_ctor_set(x_37, 9, x_35); -lean_ctor_set_uint8(x_37, sizeof(void*)*10, x_36); -x_38 = l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_expandDeclId___spec__15(x_10, x_37, x_6, x_18); -x_39 = lean_ctor_get(x_38, 0); -lean_inc(x_39); -x_40 = lean_ctor_get(x_38, 1); -lean_inc(x_40); -if (lean_is_exclusive(x_38)) { - lean_ctor_release(x_38, 0); - lean_ctor_release(x_38, 1); - x_41 = x_38; -} else { - lean_dec_ref(x_38); - x_41 = lean_box(0); -} -if (lean_is_scalar(x_41)) { - x_42 = lean_alloc_ctor(1, 2, 0); -} else { - x_42 = x_41; -} -lean_ctor_set(x_42, 0, x_39); -lean_ctor_set(x_42, 1, x_40); -return x_42; -} -} -} -else -{ -lean_object* x_43; -lean_dec(x_5); -x_43 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_43, 0, x_4); -lean_ctor_set(x_43, 1, x_7); -return x_43; -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_expandDeclId___at_Lean_Elab_Command_expandDeclId___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) { -_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; uint8_t x_22; lean_object* x_23; lean_object* x_24; -x_9 = l_Lean_Elab_Command_getRef(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 = l_Lean_replaceRef(x_1, x_10); -lean_dec(x_10); -x_13 = lean_ctor_get(x_6, 0); -lean_inc(x_13); -x_14 = lean_ctor_get(x_6, 1); -lean_inc(x_14); -x_15 = lean_ctor_get(x_6, 2); -lean_inc(x_15); -x_16 = lean_ctor_get(x_6, 3); -lean_inc(x_16); -x_17 = lean_ctor_get(x_6, 4); -lean_inc(x_17); -x_18 = lean_ctor_get(x_6, 5); -lean_inc(x_18); -x_19 = lean_ctor_get(x_6, 7); -lean_inc(x_19); -x_20 = lean_ctor_get(x_6, 8); -lean_inc(x_20); -x_21 = lean_ctor_get(x_6, 9); -lean_inc(x_21); -x_22 = lean_ctor_get_uint8(x_6, sizeof(void*)*10); -x_23 = lean_alloc_ctor(0, 10, 1); -lean_ctor_set(x_23, 0, x_13); -lean_ctor_set(x_23, 1, x_14); -lean_ctor_set(x_23, 2, x_15); -lean_ctor_set(x_23, 3, x_16); -lean_ctor_set(x_23, 4, x_17); -lean_ctor_set(x_23, 5, x_18); -lean_ctor_set(x_23, 6, x_12); -lean_ctor_set(x_23, 7, x_19); -lean_ctor_set(x_23, 8, x_20); -lean_ctor_set(x_23, 9, x_21); -lean_ctor_set_uint8(x_23, sizeof(void*)*10, x_22); -x_24 = l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2(x_2, x_3, x_4, x_23, x_7, x_11); -if (lean_obj_tag(x_24) == 0) -{ -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -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); -x_28 = lean_ctor_get(x_25, 1); -lean_inc(x_28); -lean_dec(x_25); -x_29 = lean_ctor_get(x_3, 0); -lean_inc(x_29); -lean_dec(x_3); -lean_inc(x_27); -x_30 = l_Lean_addDocString_x27___at_Lean_Elab_Command_expandDeclId___spec__13(x_27, x_29, x_6, x_7, x_26); -if (lean_obj_tag(x_30) == 0) -{ -uint8_t x_31; -x_31 = !lean_is_exclusive(x_30); -if (x_31 == 0) -{ -lean_object* x_32; lean_object* x_33; -x_32 = lean_ctor_get(x_30, 0); -lean_dec(x_32); -x_33 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_33, 0, x_28); -lean_ctor_set(x_33, 1, x_27); -lean_ctor_set(x_33, 2, x_5); -lean_ctor_set(x_30, 0, x_33); -return x_30; -} -else -{ -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_alloc_ctor(0, 3, 0); -lean_ctor_set(x_35, 0, x_28); -lean_ctor_set(x_35, 1, x_27); -lean_ctor_set(x_35, 2, x_5); -x_36 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_36, 0, x_35); -lean_ctor_set(x_36, 1, x_34); -return x_36; -} -} -else -{ -uint8_t x_37; -lean_dec(x_28); -lean_dec(x_27); -lean_dec(x_5); -x_37 = !lean_is_exclusive(x_30); -if (x_37 == 0) -{ -return x_30; -} -else -{ -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_30, 0); -x_39 = lean_ctor_get(x_30, 1); -lean_inc(x_39); -lean_inc(x_38); -lean_dec(x_30); -x_40 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_40, 0, x_38); -lean_ctor_set(x_40, 1, x_39); -return x_40; -} -} -} -else -{ -uint8_t x_41; -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -x_41 = !lean_is_exclusive(x_24); -if (x_41 == 0) -{ -return x_24; -} -else -{ -lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_ctor_get(x_24, 0); -x_43 = lean_ctor_get(x_24, 1); -lean_inc(x_43); -lean_inc(x_42); -lean_dec(x_24); -x_44 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_44, 0, x_42); -lean_ctor_set(x_44, 1, x_43); -return x_44; -} -} -} -} -static lean_object* _init_l_Lean_Elab_expandDeclId___at_Lean_Elab_Command_expandDeclId___spec__1___closed__1() { -_start: -{ -uint8_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = 1; -x_2 = l_Lean_Elab_Command_instInhabitedScope___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_EXPORT lean_object* l_Lean_Elab_expandDeclId___at_Lean_Elab_Command_expandDeclId___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; -x_8 = l_Lean_Elab_expandDeclIdCore(x_3); -x_9 = lean_ctor_get(x_8, 0); -lean_inc(x_9); -x_10 = lean_ctor_get(x_8, 1); -lean_inc(x_10); -lean_dec(x_8); -x_11 = l_Lean_Syntax_isNone(x_10); -if (x_11 == 0) -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; -x_12 = lean_unsigned_to_nat(1u); -x_13 = l_Lean_Syntax_getArg(x_10, x_12); -lean_dec(x_10); -x_14 = l_Lean_Syntax_getArgs(x_13); -lean_dec(x_13); -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) -{ -lean_object* x_35; -lean_dec(x_15); -lean_dec(x_14); -x_35 = l_Lean_Elab_Command_instInhabitedScope___closed__1; -x_18 = x_35; -goto block_34; -} -else -{ -uint8_t x_36; -x_36 = lean_nat_dec_le(x_15, x_15); -if (x_36 == 0) -{ -lean_object* x_37; -lean_dec(x_15); -lean_dec(x_14); -x_37 = l_Lean_Elab_Command_instInhabitedScope___closed__1; -x_18 = x_37; -goto block_34; -} -else -{ -size_t x_38; size_t x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_38 = 0; -x_39 = lean_usize_of_nat(x_15); -lean_dec(x_15); -x_40 = l_Lean_Elab_expandDeclId___at_Lean_Elab_Command_expandDeclId___spec__1___closed__1; -x_41 = l_Array_foldlMUnsafe_fold___at_Lean_Syntax_SepArray_getElems___spec__1(x_14, x_38, x_39, x_40); -lean_dec(x_14); -x_42 = lean_ctor_get(x_41, 1); -lean_inc(x_42); -lean_dec(x_41); -x_18 = x_42; -goto block_34; -} -} -block_34: -{ -lean_object* x_19; uint8_t x_20; -x_19 = lean_array_get_size(x_18); -x_20 = lean_nat_dec_lt(x_16, x_19); -if (x_20 == 0) -{ -lean_object* x_21; -lean_dec(x_19); -lean_dec(x_18); -x_21 = l_Lean_Elab_expandDeclId___at_Lean_Elab_Command_expandDeclId___spec__1___lambda__1(x_3, x_1, x_4, x_9, x_2, x_5, x_6, x_7); -return x_21; -} -else -{ -uint8_t x_22; -x_22 = lean_nat_dec_le(x_19, x_19); -if (x_22 == 0) -{ -lean_object* x_23; -lean_dec(x_19); -lean_dec(x_18); -x_23 = l_Lean_Elab_expandDeclId___at_Lean_Elab_Command_expandDeclId___spec__1___lambda__1(x_3, x_1, x_4, x_9, x_2, x_5, x_6, x_7); -return x_23; -} -else -{ -size_t x_24; size_t x_25; lean_object* x_26; -x_24 = 0; -x_25 = lean_usize_of_nat(x_19); -lean_dec(x_19); -lean_inc(x_5); -x_26 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_expandDeclId___spec__17(x_18, x_24, x_25, x_2, x_5, x_6, x_7); -lean_dec(x_18); -if (lean_obj_tag(x_26) == 0) -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_26, 0); -lean_inc(x_27); -x_28 = lean_ctor_get(x_26, 1); -lean_inc(x_28); -lean_dec(x_26); -x_29 = l_Lean_Elab_expandDeclId___at_Lean_Elab_Command_expandDeclId___spec__1___lambda__1(x_3, x_1, x_4, x_9, x_27, x_5, x_6, x_28); -return x_29; -} -else -{ -uint8_t x_30; -lean_dec(x_9); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_1); -x_30 = !lean_is_exclusive(x_26); -if (x_30 == 0) -{ -return x_26; -} -else -{ -lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_31 = lean_ctor_get(x_26, 0); -x_32 = lean_ctor_get(x_26, 1); -lean_inc(x_32); -lean_inc(x_31); -lean_dec(x_26); -x_33 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_33, 0, x_31); -lean_ctor_set(x_33, 1, x_32); -return x_33; -} -} -} -} -} -} -else -{ -lean_object* x_43; -lean_dec(x_10); -x_43 = l_Lean_Elab_expandDeclId___at_Lean_Elab_Command_expandDeclId___spec__1___lambda__1(x_3, x_1, x_4, x_9, x_2, x_5, x_6, x_7); -return x_43; -} -} -} -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__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; uint8_t x_11; -x_5 = l_Lean_Elab_Command_getRef(x_2, x_3, x_4); -x_6 = lean_ctor_get(x_5, 0); -lean_inc(x_6); -x_7 = lean_ctor_get(x_5, 1); -lean_inc(x_7); -lean_dec(x_5); -x_8 = lean_ctor_get(x_2, 4); -lean_inc(x_8); -lean_inc(x_8); -x_9 = l_Lean_Elab_getBetterRef(x_6, x_8); -lean_dec(x_6); -x_10 = l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1(x_1, x_2, x_3, x_7); -x_11 = !lean_is_exclusive(x_10); -if (x_11 == 0) -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; -x_12 = lean_ctor_get(x_10, 0); -x_13 = lean_ctor_get(x_10, 1); -x_14 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_12, x_8, x_2, x_3, x_13); -lean_dec(x_2); -x_15 = !lean_is_exclusive(x_14); -if (x_15 == 0) -{ -lean_object* x_16; -x_16 = lean_ctor_get(x_14, 0); -lean_ctor_set(x_10, 1, x_16); -lean_ctor_set(x_10, 0, x_9); -lean_ctor_set_tag(x_14, 1); -lean_ctor_set(x_14, 0, x_10); -return x_14; -} -else -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_14, 0); -x_18 = lean_ctor_get(x_14, 1); -lean_inc(x_18); -lean_inc(x_17); -lean_dec(x_14); -lean_ctor_set(x_10, 1, x_17); -lean_ctor_set(x_10, 0, x_9); -x_19 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_19, 0, x_10); -lean_ctor_set(x_19, 1, x_18); -return x_19; -} +lean_dec(x_63); +x_68 = l_Lean_MessageLog_toArray(x_52); +x_69 = lean_array_size(x_68); +x_70 = 0; +x_71 = l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___closed__1; +x_72 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___spec__1(x_71, x_68, x_69, x_70, x_71); +lean_dec(x_68); +x_73 = lean_ctor_get(x_72, 0); +lean_inc(x_73); +lean_dec(x_72); +if (lean_obj_tag(x_73) == 0) +{ +lean_object* x_74; +x_74 = l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___closed__3; +if (lean_obj_tag(x_74) == 0) +{ +lean_object* x_75; lean_object* x_76; +x_75 = lean_box(0); +x_76 = l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___lambda__1(x_52, x_55, x_43, x_75, x_3, x_4, x_67); +lean_dec(x_55); +return x_76; } 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; -x_20 = lean_ctor_get(x_10, 0); -x_21 = lean_ctor_get(x_10, 1); -lean_inc(x_21); -lean_inc(x_20); -lean_dec(x_10); -x_22 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_20, x_8, x_2, x_3, x_21); -lean_dec(x_2); -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -x_24 = lean_ctor_get(x_22, 1); -lean_inc(x_24); -if (lean_is_exclusive(x_22)) { - lean_ctor_release(x_22, 0); - lean_ctor_release(x_22, 1); - x_25 = x_22; -} else { - lean_dec_ref(x_22); - x_25 = lean_box(0); -} -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_9); -lean_ctor_set(x_26, 1, x_23); -if (lean_is_scalar(x_25)) { - x_27 = lean_alloc_ctor(1, 2, 0); -} else { - x_27 = x_25; - lean_ctor_set_tag(x_27, 1); -} -lean_ctor_set(x_27, 0, x_26); -lean_ctor_set(x_27, 1, x_24); -return x_27; -} -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__19___closed__1() { -_start: +lean_object* x_77; lean_object* x_78; lean_object* x_79; uint8_t x_80; +lean_dec(x_55); +lean_dec(x_52); +lean_dec(x_43); +x_77 = lean_ctor_get(x_74, 0); +lean_inc(x_77); +x_78 = lean_ctor_get(x_77, 4); +lean_inc(x_78); +lean_dec(x_77); +x_79 = l_Lean_throwError___at_Lean_realizeGlobalConstCore___spec__3(x_78, x_3, x_4, x_67); +x_80 = !lean_is_exclusive(x_79); +if (x_80 == 0) { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("', there is a section variable with the same name", 49, 49); -return x_1; -} +return x_79; } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__19___closed__2() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__19___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +lean_object* x_81; lean_object* x_82; lean_object* x_83; +x_81 = lean_ctor_get(x_79, 0); +x_82 = lean_ctor_get(x_79, 1); +lean_inc(x_82); +lean_inc(x_81); +lean_dec(x_79); +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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___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) { -_start: -{ -uint8_t x_9; -x_9 = lean_usize_dec_lt(x_4, x_3); -if (x_9 == 0) -{ -lean_object* x_10; -lean_dec(x_6); -lean_dec(x_1); -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_5); -lean_ctor_set(x_10, 1, x_8); -return x_10; } else { -lean_object* x_11; lean_object* x_12; uint8_t x_13; -lean_dec(x_5); -x_11 = lean_array_uget(x_2, x_4); -x_12 = lean_ctor_get(x_1, 0); -lean_inc(x_12); -x_13 = lean_name_eq(x_11, x_12); -lean_dec(x_11); -if (x_13 == 0) +lean_object* x_84; +x_84 = lean_ctor_get(x_73, 0); +lean_inc(x_84); +lean_dec(x_73); +if (lean_obj_tag(x_84) == 0) { -size_t x_14; size_t x_15; lean_object* x_16; -lean_dec(x_12); -x_14 = 1; -x_15 = lean_usize_add(x_4, x_14); -x_16 = lean_box(0); -x_4 = x_15; -x_5 = x_16; -goto _start; +lean_object* x_85; lean_object* x_86; +x_85 = lean_box(0); +x_86 = l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___lambda__1(x_52, x_55, x_43, x_85, x_3, x_4, x_67); +lean_dec(x_55); +return x_86; } 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; -lean_dec(x_1); -x_18 = l_Lean_MessageData_ofName(x_12); -x_19 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__2; -x_20 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_20, 0, x_19); -lean_ctor_set(x_20, 1, x_18); -x_21 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__19___closed__2; -x_22 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_22, 0, x_20); -lean_ctor_set(x_22, 1, x_21); -x_23 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__18(x_22, x_6, x_7, x_8); -x_24 = !lean_is_exclusive(x_23); -if (x_24 == 0) +lean_object* x_87; lean_object* x_88; lean_object* x_89; uint8_t x_90; +lean_dec(x_55); +lean_dec(x_52); +lean_dec(x_43); +x_87 = lean_ctor_get(x_84, 0); +lean_inc(x_87); +lean_dec(x_84); +x_88 = lean_ctor_get(x_87, 4); +lean_inc(x_88); +lean_dec(x_87); +x_89 = l_Lean_throwError___at_Lean_realizeGlobalConstCore___spec__3(x_88, x_3, x_4, x_67); +x_90 = !lean_is_exclusive(x_89); +if (x_90 == 0) { -return x_23; +return x_89; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_23, 0); -x_26 = lean_ctor_get(x_23, 1); -lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_23); -x_27 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_26); -return x_27; +lean_object* x_91; lean_object* x_92; lean_object* x_93; +x_91 = lean_ctor_get(x_89, 0); +x_92 = lean_ctor_get(x_89, 1); +lean_inc(x_92); +lean_inc(x_91); +lean_dec(x_89); +x_93 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_93, 0, x_91); +lean_ctor_set(x_93, 1, x_92); +return x_93; } } } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandDeclId(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; -x_6 = l_Lean_Elab_Command_getScope___rarg(x_4, x_5); -x_7 = lean_ctor_get(x_6, 0); -lean_inc(x_7); -x_8 = lean_ctor_get(x_6, 1); -lean_inc(x_8); -lean_dec(x_6); -x_9 = lean_ctor_get(x_7, 2); -lean_inc(x_9); -lean_dec(x_7); -x_10 = l_Lean_Elab_Command_getLevelNames___rarg(x_4, x_8); -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -x_12 = lean_ctor_get(x_10, 1); -lean_inc(x_12); -lean_dec(x_10); -lean_inc(x_3); -x_13 = l_Lean_Elab_expandDeclId___at_Lean_Elab_Command_expandDeclId___spec__1(x_9, x_11, x_1, x_2, x_3, x_4, x_12); -if (lean_obj_tag(x_13) == 0) +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; lean_object* x_23; lean_object* x_24; -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_Command_getScope___rarg(x_4, 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, 5); -lean_inc(x_19); -lean_dec(x_17); -x_20 = lean_array_get_size(x_19); -x_21 = lean_unsigned_to_nat(0u); -x_22 = lean_nat_dec_lt(x_21, x_20); -if (x_22 == 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; +x_94 = lean_ctor_get(x_49, 3); +x_95 = lean_ctor_get(x_49, 4); +x_96 = lean_ctor_get(x_49, 5); +x_97 = lean_ctor_get(x_49, 6); +lean_inc(x_97); +lean_inc(x_96); +lean_inc(x_95); +lean_inc(x_94); +lean_dec(x_49); +x_98 = l_Lean_PersistentArray_append___rarg(x_94, x_56); +lean_dec(x_56); +x_99 = lean_alloc_ctor(0, 7, 0); +lean_ctor_set(x_99, 0, x_51); +lean_ctor_set(x_99, 1, x_53); +lean_ctor_set(x_99, 2, x_54); +lean_ctor_set(x_99, 3, x_98); +lean_ctor_set(x_99, 4, x_95); +lean_ctor_set(x_99, 5, x_96); +lean_ctor_set(x_99, 6, x_97); +x_100 = lean_st_ref_set(x_4, x_99, x_50); +if (x_2 == 0) { -lean_object* x_38; -lean_dec(x_20); -lean_dec(x_19); -x_38 = l_Lean_Elab_Command_instInhabitedScope___closed__1; -x_23 = x_38; -x_24 = x_18; -goto block_37; +lean_object* x_101; lean_object* x_102; lean_object* x_103; +x_101 = lean_ctor_get(x_100, 1); +lean_inc(x_101); +lean_dec(x_100); +x_102 = lean_box(0); +x_103 = l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___lambda__1(x_52, x_55, x_43, x_102, x_3, x_4, x_101); +lean_dec(x_55); +return x_103; } else { -uint8_t x_39; -x_39 = lean_nat_dec_le(x_20, x_20); -if (x_39 == 0) +lean_object* x_104; lean_object* x_105; size_t x_106; size_t x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; +x_104 = lean_ctor_get(x_100, 1); +lean_inc(x_104); +lean_dec(x_100); +x_105 = l_Lean_MessageLog_toArray(x_52); +x_106 = lean_array_size(x_105); +x_107 = 0; +x_108 = l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___closed__1; +x_109 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___spec__1(x_108, x_105, x_106, x_107, x_108); +lean_dec(x_105); +x_110 = lean_ctor_get(x_109, 0); +lean_inc(x_110); +lean_dec(x_109); +if (lean_obj_tag(x_110) == 0) { -lean_object* x_40; -lean_dec(x_20); -lean_dec(x_19); -x_40 = l_Lean_Elab_Command_instInhabitedScope___closed__1; -x_23 = x_40; -x_24 = x_18; -goto block_37; +lean_object* x_111; +x_111 = l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___closed__3; +if (lean_obj_tag(x_111) == 0) +{ +lean_object* x_112; lean_object* x_113; +x_112 = lean_box(0); +x_113 = l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___lambda__1(x_52, x_55, x_43, x_112, x_3, x_4, x_104); +lean_dec(x_55); +return x_113; } 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_20); -lean_dec(x_20); -x_43 = l_Lean_Elab_Command_instInhabitedScope___closed__1; -x_44 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Command_0__Lean_Elab_Command_mkTermContext___spec__2(x_19, x_41, x_42, x_43, x_3, x_4, x_18); -lean_dec(x_19); -if (lean_obj_tag(x_44) == 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_23 = x_45; -x_24 = x_46; -goto block_37; +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_dec(x_55); +lean_dec(x_52); +lean_dec(x_43); +x_114 = lean_ctor_get(x_111, 0); +lean_inc(x_114); +x_115 = lean_ctor_get(x_114, 4); +lean_inc(x_115); +lean_dec(x_114); +x_116 = l_Lean_throwError___at_Lean_realizeGlobalConstCore___spec__3(x_115, x_3, x_4, x_104); +x_117 = lean_ctor_get(x_116, 0); +lean_inc(x_117); +x_118 = lean_ctor_get(x_116, 1); +lean_inc(x_118); +if (lean_is_exclusive(x_116)) { + lean_ctor_release(x_116, 0); + lean_ctor_release(x_116, 1); + x_119 = x_116; +} else { + lean_dec_ref(x_116); + x_119 = lean_box(0); +} +if (lean_is_scalar(x_119)) { + x_120 = lean_alloc_ctor(1, 2, 0); +} else { + x_120 = x_119; +} +lean_ctor_set(x_120, 0, x_117); +lean_ctor_set(x_120, 1, x_118); +return x_120; +} } else { -uint8_t x_47; -lean_dec(x_14); -lean_dec(x_3); -x_47 = !lean_is_exclusive(x_44); -if (x_47 == 0) +lean_object* x_121; +x_121 = lean_ctor_get(x_110, 0); +lean_inc(x_121); +lean_dec(x_110); +if (lean_obj_tag(x_121) == 0) { -return x_44; +lean_object* x_122; lean_object* x_123; +x_122 = lean_box(0); +x_123 = l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___lambda__1(x_52, x_55, x_43, x_122, x_3, x_4, x_104); +lean_dec(x_55); +return x_123; } 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_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_dec(x_55); +lean_dec(x_52); +lean_dec(x_43); +x_124 = lean_ctor_get(x_121, 0); +lean_inc(x_124); +lean_dec(x_121); +x_125 = lean_ctor_get(x_124, 4); +lean_inc(x_125); +lean_dec(x_124); +x_126 = l_Lean_throwError___at_Lean_realizeGlobalConstCore___spec__3(x_125, x_3, x_4, x_104); +x_127 = lean_ctor_get(x_126, 0); +lean_inc(x_127); +x_128 = lean_ctor_get(x_126, 1); +lean_inc(x_128); +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_126); + x_129 = lean_box(0); } +if (lean_is_scalar(x_129)) { + x_130 = lean_alloc_ctor(1, 2, 0); +} else { + x_130 = x_129; } +lean_ctor_set(x_130, 0, x_127); +lean_ctor_set(x_130, 1, x_128); +return x_130; } } -block_37: -{ -size_t x_25; size_t x_26; lean_object* x_27; lean_object* x_28; -x_25 = lean_array_size(x_23); -x_26 = 0; -x_27 = lean_box(0); -lean_inc(x_14); -x_28 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__19(x_14, x_23, x_25, x_26, x_27, x_3, x_4, x_24); -lean_dec(x_23); -if (lean_obj_tag(x_28) == 0) -{ -uint8_t x_29; -x_29 = !lean_is_exclusive(x_28); -if (x_29 == 0) -{ -lean_object* x_30; -x_30 = lean_ctor_get(x_28, 0); -lean_dec(x_30); -lean_ctor_set(x_28, 0, x_14); -return x_28; } -else -{ -lean_object* x_31; lean_object* x_32; -x_31 = lean_ctor_get(x_28, 1); -lean_inc(x_31); -lean_dec(x_28); -x_32 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_32, 0, x_14); -lean_ctor_set(x_32, 1, x_31); -return x_32; } } else { -uint8_t x_33; -lean_dec(x_14); -x_33 = !lean_is_exclusive(x_28); -if (x_33 == 0) +uint8_t x_131; +lean_dec(x_40); +x_131 = !lean_is_exclusive(x_42); +if (x_131 == 0) { -return x_28; +return x_42; } 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_object* x_132; lean_object* x_133; lean_object* x_134; +x_132 = lean_ctor_get(x_42, 0); +x_133 = lean_ctor_get(x_42, 1); +lean_inc(x_133); +lean_inc(x_132); +lean_dec(x_42); +x_134 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_134, 0, x_132); +lean_ctor_set(x_134, 1, x_133); +return x_134; } } } +else +{ +uint8_t x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; +x_135 = lean_ctor_get_uint8(x_26, sizeof(void*)*2); +lean_dec(x_26); +x_136 = l_Lean_Elab_Command_mkState___closed__8; +x_137 = l_Lean_Elab_Command_mkState___closed__11; +x_138 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_138, 0, x_136); +lean_ctor_set(x_138, 1, x_137); +lean_ctor_set_uint8(x_138, sizeof(void*)*2, x_135); +x_139 = l___private_Lean_Elab_Command_0__Lean_Elab_Command_runCore___rarg___closed__4; +lean_inc(x_14); +x_140 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_140, 0, x_23); +lean_ctor_set(x_140, 1, x_139); +lean_ctor_set(x_140, 2, x_6); +lean_ctor_set(x_140, 3, x_24); +lean_ctor_set(x_140, 4, x_14); +lean_ctor_set(x_140, 5, x_25); +lean_ctor_set(x_140, 6, x_138); +lean_ctor_set(x_140, 7, x_137); +x_141 = lean_st_mk_ref(x_140, x_9); +x_142 = lean_ctor_get(x_141, 0); +lean_inc(x_142); +x_143 = lean_ctor_get(x_141, 1); +lean_inc(x_143); +lean_dec(x_141); +lean_inc(x_142); +x_144 = lean_apply_3(x_1, x_22, x_142, x_143); +if (lean_obj_tag(x_144) == 0) +{ +lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; 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_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_st_ref_get(x_142, x_146); +lean_dec(x_142); +x_148 = lean_ctor_get(x_147, 0); +lean_inc(x_148); +x_149 = lean_ctor_get(x_147, 1); +lean_inc(x_149); +lean_dec(x_147); +x_150 = lean_st_ref_take(x_4, x_149); +x_151 = lean_ctor_get(x_150, 0); +lean_inc(x_151); +x_152 = lean_ctor_get(x_150, 1); +lean_inc(x_152); +lean_dec(x_150); +x_153 = lean_ctor_get(x_148, 0); +lean_inc(x_153); +x_154 = lean_ctor_get(x_148, 1); +lean_inc(x_154); +x_155 = lean_ctor_get(x_148, 3); +lean_inc(x_155); +x_156 = lean_ctor_get(x_148, 5); +lean_inc(x_156); +x_157 = lean_ctor_get(x_148, 6); +lean_inc(x_157); +x_158 = lean_ctor_get(x_148, 7); +lean_inc(x_158); +lean_dec(x_148); +x_159 = lean_ctor_get(x_151, 3); +lean_inc(x_159); +x_160 = lean_ctor_get(x_151, 4); +lean_inc(x_160); +x_161 = lean_ctor_get(x_151, 5); +lean_inc(x_161); +x_162 = lean_ctor_get(x_151, 6); +lean_inc(x_162); +if (lean_is_exclusive(x_151)) { + lean_ctor_release(x_151, 0); + lean_ctor_release(x_151, 1); + lean_ctor_release(x_151, 2); + lean_ctor_release(x_151, 3); + lean_ctor_release(x_151, 4); + lean_ctor_release(x_151, 5); + lean_ctor_release(x_151, 6); + x_163 = x_151; +} else { + lean_dec_ref(x_151); + x_163 = lean_box(0); +} +x_164 = l_Lean_PersistentArray_append___rarg(x_159, x_158); +lean_dec(x_158); +if (lean_is_scalar(x_163)) { + x_165 = lean_alloc_ctor(0, 7, 0); +} else { + x_165 = x_163; +} +lean_ctor_set(x_165, 0, x_153); +lean_ctor_set(x_165, 1, x_155); +lean_ctor_set(x_165, 2, x_156); +lean_ctor_set(x_165, 3, x_164); +lean_ctor_set(x_165, 4, x_160); +lean_ctor_set(x_165, 5, x_161); +lean_ctor_set(x_165, 6, x_162); +x_166 = lean_st_ref_set(x_4, x_165, x_152); +if (x_2 == 0) +{ +lean_object* x_167; lean_object* x_168; lean_object* x_169; +x_167 = lean_ctor_get(x_166, 1); +lean_inc(x_167); +lean_dec(x_166); +x_168 = lean_box(0); +x_169 = l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___lambda__1(x_154, x_157, x_145, x_168, x_3, x_4, x_167); +lean_dec(x_157); +return x_169; } else { -uint8_t x_51; -lean_dec(x_3); -x_51 = !lean_is_exclusive(x_13); -if (x_51 == 0) +lean_object* x_170; lean_object* x_171; size_t x_172; size_t x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; +x_170 = lean_ctor_get(x_166, 1); +lean_inc(x_170); +lean_dec(x_166); +x_171 = l_Lean_MessageLog_toArray(x_154); +x_172 = lean_array_size(x_171); +x_173 = 0; +x_174 = l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___closed__1; +x_175 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___spec__1(x_174, x_171, x_172, x_173, x_174); +lean_dec(x_171); +x_176 = lean_ctor_get(x_175, 0); +lean_inc(x_176); +lean_dec(x_175); +if (lean_obj_tag(x_176) == 0) { -return x_13; +lean_object* x_177; +x_177 = l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___closed__3; +if (lean_obj_tag(x_177) == 0) +{ +lean_object* x_178; lean_object* x_179; +x_178 = lean_box(0); +x_179 = l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___lambda__1(x_154, x_157, x_145, x_178, x_3, x_4, x_170); +lean_dec(x_157); +return x_179; } else { -lean_object* x_52; lean_object* x_53; lean_object* x_54; -x_52 = lean_ctor_get(x_13, 0); -x_53 = lean_ctor_get(x_13, 1); -lean_inc(x_53); -lean_inc(x_52); -lean_dec(x_13); -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_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_157); +lean_dec(x_154); +lean_dec(x_145); +x_180 = lean_ctor_get(x_177, 0); +lean_inc(x_180); +x_181 = lean_ctor_get(x_180, 4); +lean_inc(x_181); +lean_dec(x_180); +x_182 = l_Lean_throwError___at_Lean_realizeGlobalConstCore___spec__3(x_181, x_3, x_4, x_170); +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_182); + x_185 = lean_box(0); } +if (lean_is_scalar(x_185)) { + x_186 = lean_alloc_ctor(1, 2, 0); +} else { + x_186 = x_185; } +lean_ctor_set(x_186, 0, x_183); +lean_ctor_set(x_186, 1, x_184); +return x_186; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4___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_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_1, x_2, x_3, x_4); -lean_dec(x_3); -return x_5; -} +lean_object* x_187; +x_187 = lean_ctor_get(x_176, 0); +lean_inc(x_187); +lean_dec(x_176); +if (lean_obj_tag(x_187) == 0) +{ +lean_object* x_188; lean_object* x_189; +x_188 = lean_box(0); +x_189 = l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___lambda__1(x_154, x_157, x_145, x_188, x_3, x_4, x_170); +lean_dec(x_157); +return x_189; } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___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: +else { -size_t x_10; size_t x_11; lean_object* x_12; -x_10 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_11 = lean_unbox_usize(x_5); -lean_dec(x_5); -x_12 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5(x_1, x_2, x_3, x_10, x_11, x_6, x_7, x_8, x_9); -lean_dec(x_8); -lean_dec(x_3); -return x_12; +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_dec(x_157); +lean_dec(x_154); +lean_dec(x_145); +x_190 = lean_ctor_get(x_187, 0); +lean_inc(x_190); +lean_dec(x_187); +x_191 = lean_ctor_get(x_190, 4); +lean_inc(x_191); +lean_dec(x_190); +x_192 = l_Lean_throwError___at_Lean_realizeGlobalConstCore___spec__3(x_191, x_3, x_4, x_170); +x_193 = lean_ctor_get(x_192, 0); +lean_inc(x_193); +x_194 = lean_ctor_get(x_192, 1); +lean_inc(x_194); +if (lean_is_exclusive(x_192)) { + lean_ctor_release(x_192, 0); + lean_ctor_release(x_192, 1); + x_195 = x_192; +} else { + lean_dec_ref(x_192); + x_195 = lean_box(0); } +if (lean_is_scalar(x_195)) { + x_196 = lean_alloc_ctor(1, 2, 0); +} else { + x_196 = x_195; } -LEAN_EXPORT lean_object* l_Lean_Elab_checkIfShadowingStructureField___at_Lean_Elab_Command_expandDeclId___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -lean_object* x_5; -x_5 = l_Lean_Elab_checkIfShadowingStructureField___at_Lean_Elab_Command_expandDeclId___spec__3(x_1, x_2, x_3, x_4); -lean_dec(x_3); -return x_5; +lean_ctor_set(x_196, 0, x_193); +lean_ctor_set(x_196, 1, x_194); +return x_196; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___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_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__10(x_1, x_2, x_3, x_4); -lean_dec(x_3); -return x_5; } } -LEAN_EXPORT lean_object* l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9___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_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9(x_1, x_2, x_3, x_4); -lean_dec(x_3); -return x_5; +lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; +lean_dec(x_142); +x_197 = lean_ctor_get(x_144, 0); +lean_inc(x_197); +x_198 = lean_ctor_get(x_144, 1); +lean_inc(x_198); +if (lean_is_exclusive(x_144)) { + lean_ctor_release(x_144, 0); + lean_ctor_release(x_144, 1); + x_199 = x_144; +} else { + lean_dec_ref(x_144); + x_199 = lean_box(0); } +if (lean_is_scalar(x_199)) { + x_200 = lean_alloc_ctor(1, 2, 0); +} else { + x_200 = x_199; } -LEAN_EXPORT lean_object* l_Lean_mkConstWithLevelParams___at_Lean_Elab_Command_expandDeclId___spec__8___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_mkConstWithLevelParams___at_Lean_Elab_Command_expandDeclId___spec__8(x_1, x_2, x_3, x_4); -lean_dec(x_3); -return x_5; +lean_ctor_set(x_200, 0, x_197); +lean_ctor_set(x_200, 1, x_198); +return x_200; } } -LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoTree___at_Lean_Elab_Command_expandDeclId___spec__12___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_Elab_pushInfoTree___at_Lean_Elab_Command_expandDeclId___spec__12(x_1, x_2, x_3, x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_5; +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; 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; uint8_t x_223; lean_object* x_224; lean_object* x_225; uint8_t x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; +x_201 = lean_ctor_get(x_6, 0); +x_202 = lean_ctor_get(x_6, 1); +lean_inc(x_202); +lean_inc(x_201); +lean_dec(x_6); +x_203 = lean_ctor_get(x_3, 0); +x_204 = lean_ctor_get(x_3, 1); +x_205 = lean_ctor_get(x_3, 2); +x_206 = lean_ctor_get(x_3, 3); +x_207 = lean_ctor_get(x_3, 4); +x_208 = lean_ctor_get(x_3, 5); +x_209 = lean_ctor_get(x_3, 10); +x_210 = lean_ctor_get(x_3, 11); +x_211 = lean_ctor_get_uint8(x_3, sizeof(void*)*12 + 1); +x_212 = lean_box(0); +x_213 = lean_box(0); +x_214 = lean_unsigned_to_nat(0u); +lean_inc(x_210); +lean_inc(x_208); +lean_inc(x_209); +lean_inc(x_206); +lean_inc(x_204); +lean_inc(x_203); +x_215 = lean_alloc_ctor(0, 10, 1); +lean_ctor_set(x_215, 0, x_203); +lean_ctor_set(x_215, 1, x_204); +lean_ctor_set(x_215, 2, x_206); +lean_ctor_set(x_215, 3, x_214); +lean_ctor_set(x_215, 4, x_212); +lean_ctor_set(x_215, 5, x_209); +lean_ctor_set(x_215, 6, x_208); +lean_ctor_set(x_215, 7, x_213); +lean_ctor_set(x_215, 8, x_213); +lean_ctor_set(x_215, 9, x_210); +lean_ctor_set_uint8(x_215, sizeof(void*)*10, x_211); +x_216 = lean_ctor_get(x_201, 0); +lean_inc(x_216); +x_217 = lean_ctor_get(x_201, 1); +lean_inc(x_217); +x_218 = lean_ctor_get(x_201, 2); +lean_inc(x_218); +x_219 = lean_ctor_get(x_201, 6); +lean_inc(x_219); +lean_dec(x_201); +x_220 = l_Lean_Elab_Command_instInhabitedScope___closed__2; +x_221 = lean_box(0); +x_222 = l_Lean_Elab_Command_mkState___closed__1; +x_223 = 0; +lean_inc(x_205); +x_224 = lean_alloc_ctor(0, 9, 1); +lean_ctor_set(x_224, 0, x_220); +lean_ctor_set(x_224, 1, x_205); +lean_ctor_set(x_224, 2, x_221); +lean_ctor_set(x_224, 3, x_212); +lean_ctor_set(x_224, 4, x_212); +lean_ctor_set(x_224, 5, x_222); +lean_ctor_set(x_224, 6, x_222); +lean_ctor_set(x_224, 7, x_212); +lean_ctor_set(x_224, 8, x_212); +lean_ctor_set_uint8(x_224, sizeof(void*)*9, x_223); +x_225 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_225, 0, x_224); +lean_ctor_set(x_225, 1, x_212); +x_226 = lean_ctor_get_uint8(x_219, sizeof(void*)*2); +if (lean_is_exclusive(x_219)) { + lean_ctor_release(x_219, 0); + lean_ctor_release(x_219, 1); + x_227 = x_219; +} else { + lean_dec_ref(x_219); + x_227 = lean_box(0); } +x_228 = l_Lean_Elab_Command_mkState___closed__8; +x_229 = l_Lean_Elab_Command_mkState___closed__11; +if (lean_is_scalar(x_227)) { + x_230 = lean_alloc_ctor(0, 2, 1); +} else { + x_230 = x_227; } -LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_expandDeclId___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: +lean_ctor_set(x_230, 0, x_228); +lean_ctor_set(x_230, 1, x_229); +lean_ctor_set_uint8(x_230, sizeof(void*)*2, x_226); +x_231 = l___private_Lean_Elab_Command_0__Lean_Elab_Command_runCore___rarg___closed__4; +lean_inc(x_207); +x_232 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_232, 0, x_216); +lean_ctor_set(x_232, 1, x_231); +lean_ctor_set(x_232, 2, x_225); +lean_ctor_set(x_232, 3, x_217); +lean_ctor_set(x_232, 4, x_207); +lean_ctor_set(x_232, 5, x_218); +lean_ctor_set(x_232, 6, x_230); +lean_ctor_set(x_232, 7, x_229); +x_233 = lean_st_mk_ref(x_232, x_202); +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); +lean_inc(x_234); +x_236 = lean_apply_3(x_1, x_215, x_234, x_235); +if (lean_obj_tag(x_236) == 0) +{ +lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; 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; +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_st_ref_get(x_234, x_238); +lean_dec(x_234); +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_st_ref_take(x_4, x_241); +x_243 = lean_ctor_get(x_242, 0); +lean_inc(x_243); +x_244 = lean_ctor_get(x_242, 1); +lean_inc(x_244); +lean_dec(x_242); +x_245 = lean_ctor_get(x_240, 0); +lean_inc(x_245); +x_246 = lean_ctor_get(x_240, 1); +lean_inc(x_246); +x_247 = lean_ctor_get(x_240, 3); +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); +lean_dec(x_240); +x_251 = lean_ctor_get(x_243, 3); +lean_inc(x_251); +x_252 = lean_ctor_get(x_243, 4); +lean_inc(x_252); +x_253 = lean_ctor_get(x_243, 5); +lean_inc(x_253); +x_254 = lean_ctor_get(x_243, 6); +lean_inc(x_254); +if (lean_is_exclusive(x_243)) { + lean_ctor_release(x_243, 0); + lean_ctor_release(x_243, 1); + lean_ctor_release(x_243, 2); + lean_ctor_release(x_243, 3); + lean_ctor_release(x_243, 4); + lean_ctor_release(x_243, 5); + lean_ctor_release(x_243, 6); + x_255 = x_243; +} else { + lean_dec_ref(x_243); + x_255 = lean_box(0); +} +x_256 = l_Lean_PersistentArray_append___rarg(x_251, x_250); +lean_dec(x_250); +if (lean_is_scalar(x_255)) { + x_257 = lean_alloc_ctor(0, 7, 0); +} else { + x_257 = x_255; +} +lean_ctor_set(x_257, 0, x_245); +lean_ctor_set(x_257, 1, x_247); +lean_ctor_set(x_257, 2, x_248); +lean_ctor_set(x_257, 3, x_256); +lean_ctor_set(x_257, 4, x_252); +lean_ctor_set(x_257, 5, x_253); +lean_ctor_set(x_257, 6, x_254); +x_258 = lean_st_ref_set(x_4, x_257, x_244); +if (x_2 == 0) { -lean_object* x_5; -x_5 = l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_expandDeclId___spec__11(x_1, x_2, x_3, x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_5; -} +lean_object* x_259; lean_object* x_260; lean_object* x_261; +x_259 = lean_ctor_get(x_258, 1); +lean_inc(x_259); +lean_dec(x_258); +x_260 = lean_box(0); +x_261 = l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___lambda__1(x_246, x_249, x_237, x_260, x_3, x_4, x_259); +lean_dec(x_249); +return x_261; } -LEAN_EXPORT lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___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) { -_start: +else { -lean_object* x_7; -x_7 = l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6); -lean_dec(x_5); -lean_dec(x_3); -return x_7; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: +lean_object* x_262; lean_object* x_263; size_t x_264; size_t x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; +x_262 = lean_ctor_get(x_258, 1); +lean_inc(x_262); +lean_dec(x_258); +x_263 = l_Lean_MessageLog_toArray(x_246); +x_264 = lean_array_size(x_263); +x_265 = 0; +x_266 = l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___closed__1; +x_267 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___spec__1(x_266, x_263, x_264, x_265, x_266); +lean_dec(x_263); +x_268 = lean_ctor_get(x_267, 0); +lean_inc(x_268); +lean_dec(x_267); +if (lean_obj_tag(x_268) == 0) { -lean_object* x_7; -x_7 = l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6); -lean_dec(x_5); -lean_dec(x_3); -return x_7; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___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_269; +x_269 = l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___closed__3; +if (lean_obj_tag(x_269) == 0) { -lean_object* x_7; -x_7 = l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6); -lean_dec(x_5); -lean_dec(x_3); -return x_7; -} +lean_object* x_270; lean_object* x_271; +x_270 = lean_box(0); +x_271 = l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___lambda__1(x_246, x_249, x_237, x_270, x_3, x_4, x_262); +lean_dec(x_249); +return x_271; } -LEAN_EXPORT lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___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_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7(x_1, x_2, x_3, x_4); -lean_dec(x_3); -return x_5; +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_dec(x_249); +lean_dec(x_246); +lean_dec(x_237); +x_272 = lean_ctor_get(x_269, 0); +lean_inc(x_272); +x_273 = lean_ctor_get(x_272, 4); +lean_inc(x_273); +lean_dec(x_272); +x_274 = l_Lean_throwError___at_Lean_realizeGlobalConstCore___spec__3(x_273, x_3, x_4, x_262); +x_275 = lean_ctor_get(x_274, 0); +lean_inc(x_275); +x_276 = lean_ctor_get(x_274, 1); +lean_inc(x_276); +if (lean_is_exclusive(x_274)) { + lean_ctor_release(x_274, 0); + lean_ctor_release(x_274, 1); + 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, 2, 0); +} else { + x_278 = x_277; } -LEAN_EXPORT lean_object* l_Lean_Elab_applyVisibility___at_Lean_Elab_Command_expandDeclId___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -uint8_t x_6; lean_object* x_7; -x_6 = lean_unbox(x_1); -lean_dec(x_1); -x_7 = l_Lean_Elab_applyVisibility___at_Lean_Elab_Command_expandDeclId___spec__6(x_6, x_2, x_3, x_4, x_5); -lean_dec(x_4); -return x_7; +lean_ctor_set(x_278, 0, x_275); +lean_ctor_set(x_278, 1, x_276); +return x_278; } } -LEAN_EXPORT lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___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: +else { -lean_object* x_7; -x_7 = l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -return x_7; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: +lean_object* x_279; +x_279 = lean_ctor_get(x_268, 0); +lean_inc(x_279); +lean_dec(x_268); +if (lean_obj_tag(x_279) == 0) { -lean_object* x_9; -x_9 = l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_7); -lean_dec(x_5); -lean_dec(x_2); -return x_9; +lean_object* x_280; lean_object* x_281; +x_280 = lean_box(0); +x_281 = l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___lambda__1(x_246, x_249, x_237, x_280, x_3, x_4, x_262); +lean_dec(x_249); +return x_281; } -} -LEAN_EXPORT lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: +else { -uint8_t x_12; lean_object* x_13; -x_12 = lean_unbox(x_5); -lean_dec(x_5); -x_13 = l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___lambda__3(x_1, x_2, x_3, x_4, x_12, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_10); -lean_dec(x_8); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -return x_13; +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_dec(x_249); +lean_dec(x_246); +lean_dec(x_237); +x_282 = lean_ctor_get(x_279, 0); +lean_inc(x_282); +lean_dec(x_279); +x_283 = lean_ctor_get(x_282, 4); +lean_inc(x_283); +lean_dec(x_282); +x_284 = l_Lean_throwError___at_Lean_realizeGlobalConstCore___spec__3(x_283, x_3, x_4, x_262); +x_285 = lean_ctor_get(x_284, 0); +lean_inc(x_285); +x_286 = lean_ctor_get(x_284, 1); +lean_inc(x_286); +if (lean_is_exclusive(x_284)) { + lean_ctor_release(x_284, 0); + lean_ctor_release(x_284, 1); + x_287 = x_284; +} else { + lean_dec_ref(x_284); + 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_EXPORT lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -lean_object* x_7; -x_7 = l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2(x_1, x_2, x_3, x_4, x_5, x_6); -lean_dec(x_5); -lean_dec(x_2); -return x_7; +lean_ctor_set(x_288, 0, x_285); +lean_ctor_set(x_288, 1, x_286); +return x_288; } } -LEAN_EXPORT lean_object* l_Lean_addDocString___at_Lean_Elab_Command_expandDeclId___spec__14___lambda__1___boxed(lean_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_addDocString___at_Lean_Elab_Command_expandDeclId___spec__14___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_addDocString___at_Lean_Elab_Command_expandDeclId___spec__14___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_addDocString___at_Lean_Elab_Command_expandDeclId___spec__14(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_4); -return x_6; +lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; +lean_dec(x_234); +x_289 = lean_ctor_get(x_236, 0); +lean_inc(x_289); +x_290 = lean_ctor_get(x_236, 1); +lean_inc(x_290); +if (lean_is_exclusive(x_236)) { + lean_ctor_release(x_236, 0); + lean_ctor_release(x_236, 1); + x_291 = x_236; +} else { + lean_dec_ref(x_236); + 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_EXPORT lean_object* l_Lean_addDocString_x27___at_Lean_Elab_Command_expandDeclId___spec__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; -x_6 = l_Lean_addDocString_x27___at_Lean_Elab_Command_expandDeclId___spec__13(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_4); -return x_6; +lean_ctor_set(x_292, 0, x_289); +lean_ctor_set(x_292, 1, x_290); +return x_292; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___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_expandDeclId___spec__16(x_1, x_2, x_3, x_4); -lean_dec(x_3); -return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_expandDeclId___spec__15___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore(lean_object* x_1) { _start: { -lean_object* x_5; -x_5 = l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_expandDeclId___spec__15(x_1, x_2, x_3, x_4); -lean_dec(x_3); -return x_5; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___boxed), 5, 0); +return x_2; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_expandDeclId___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___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_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); +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); lean_dec(x_3); -x_10 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_expandDeclId___spec__17(x_1, x_8, x_9, x_4, x_5, x_6, x_7); -lean_dec(x_6); -lean_dec(x_1); -return x_10; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_expandDeclId___at_Lean_Elab_Command_expandDeclId___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; -x_9 = l_Lean_Elab_expandDeclId___at_Lean_Elab_Command_expandDeclId___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_7); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___spec__1(x_1, x_2, x_6, x_7, x_5); +lean_dec(x_5); +lean_dec(x_2); lean_dec(x_1); -return x_9; +return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_expandDeclId___at_Lean_Elab_Command_expandDeclId___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; -x_8 = l_Lean_Elab_expandDeclId___at_Lean_Elab_Command_expandDeclId___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_6); -lean_dec(x_3); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__18___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___lambda__2___boxed(lean_object* x_1) { _start: { -lean_object* x_5; -x_5 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__18(x_1, x_2, x_3, x_4); -lean_dec(x_3); -return x_5; +lean_object* x_2; +x_2 = l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___lambda__2(x_1); +lean_dec(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__19___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___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_9; size_t x_10; lean_object* x_11; -x_9 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_10 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_11 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__19(x_1, x_2, x_9, x_10, x_5, x_6, x_7, x_8); -lean_dec(x_7); +uint8_t x_6; lean_object* x_7; +x_6 = lean_unbox(x_2); lean_dec(x_2); -return x_11; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandDeclId___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; -x_6 = l_Lean_Elab_Command_expandDeclId(x_1, x_2, x_3, x_4, x_5); +x_7 = l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg(x_1, x_6, x_3, x_4, x_5); lean_dec(x_4); -lean_dec(x_1); -return x_6; +lean_dec(x_3); +return x_7; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_liftCommandElabM___spec__1(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_MonadExcept_ofExcept___at_Lean_liftCommandElabM___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -uint8_t x_6; -x_6 = lean_usize_dec_lt(x_4, x_3); -if (x_6 == 0) +if (lean_obj_tag(x_1) == 0) { +lean_object* x_5; lean_object* x_6; +x_5 = lean_ctor_get(x_1, 0); lean_inc(x_5); -return x_5; -} -else -{ -lean_object* x_7; uint8_t x_8; lean_object* x_9; -x_7 = lean_array_uget(x_2, x_4); -x_8 = lean_ctor_get_uint8(x_7, sizeof(void*)*5 + 1); -x_9 = lean_box(x_8); -if (lean_obj_tag(x_9) == 2) -{ -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_10 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_10, 0, x_7); -x_11 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_11, 0, x_10); -x_12 = lean_box(0); -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; +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 { -size_t x_14; size_t x_15; -lean_dec(x_9); -lean_dec(x_7); -x_14 = 1; -x_15 = lean_usize_add(x_4, x_14); -{ -size_t _tmp_3 = x_15; -lean_object* _tmp_4 = x_1; -x_4 = _tmp_3; -x_5 = _tmp_4; -} -goto _start; -} +lean_object* x_7; lean_object* x_8; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +x_8 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_8, 0, x_7); +lean_ctor_set(x_8, 1, x_4); +return x_8; } } } -LEAN_EXPORT lean_object* l_Lean_liftCommandElabM___rarg___lambda__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_liftCommandElabM___spec__1(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_box(0); +x_2 = lean_alloc_closure((void*)(l_MonadExcept_ofExcept___at_Lean_liftCommandElabM___spec__1___rarg___boxed), 4, 0); return x_2; } } -static lean_object* _init_l_Lean_liftCommandElabM___rarg___closed__1() { -_start: -{ -uint8_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = 1; -x_2 = l_Lean_Elab_Command_mkState___closed__8; -x_3 = l_Lean_Elab_Command_mkState___closed__11; -x_4 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_4, 0, x_2); -lean_ctor_set(x_4, 1, x_3); -lean_ctor_set_uint8(x_4, sizeof(void*)*2, x_1); -return x_4; -} -} -static lean_object* _init_l_Lean_liftCommandElabM___rarg___closed__2() { +LEAN_EXPORT lean_object* l_Lean_liftCommandElabM___rarg___lambda__1(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 = 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_liftCommandElabM___rarg___closed__3() { -_start: +lean_object* x_5; +x_5 = lean_apply_3(x_1, x_2, x_3, x_4); +if (lean_obj_tag(x_5) == 0) { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_liftCommandElabM___rarg___lambda__1___boxed), 1, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_liftCommandElabM___rarg___closed__4() { -_start: +uint8_t x_6; +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_liftCommandElabM___rarg___closed__3; -x_2 = lean_box(0); -x_3 = lean_apply_1(x_1, x_2); -return x_3; -} +lean_object* x_7; lean_object* x_8; +x_7 = lean_ctor_get(x_5, 0); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_7); +lean_ctor_set(x_5, 0, x_8); +return x_5; } -LEAN_EXPORT lean_object* l_Lean_liftCommandElabM___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_5 = lean_ctor_get(x_2, 0); -x_6 = lean_ctor_get(x_2, 1); -x_7 = lean_ctor_get(x_2, 2); -x_8 = lean_ctor_get(x_2, 4); -x_9 = lean_ctor_get(x_2, 5); -x_10 = lean_ctor_get(x_2, 11); -x_11 = lean_st_ref_get(x_3, x_4); -x_12 = !lean_is_exclusive(x_11); -if (x_12 == 0) +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; 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; 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_13 = lean_ctor_get(x_11, 0); -x_14 = lean_ctor_get(x_11, 1); -x_15 = lean_ctor_get(x_13, 0); -lean_inc(x_15); -lean_dec(x_13); -x_16 = lean_box(0); -x_17 = lean_box(0); -x_18 = lean_unsigned_to_nat(0u); -x_19 = l_Lean_firstFrontendMacroScope; -x_20 = 0; +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_inc(x_6); -lean_inc(x_5); -x_21 = lean_alloc_ctor(0, 10, 1); -lean_ctor_set(x_21, 0, x_5); -lean_ctor_set(x_21, 1, x_6); -lean_ctor_set(x_21, 2, x_18); -lean_ctor_set(x_21, 3, x_18); -lean_ctor_set(x_21, 4, x_16); -lean_ctor_set(x_21, 5, x_19); -lean_ctor_set(x_21, 6, x_9); -lean_ctor_set(x_21, 7, x_17); -lean_ctor_set(x_21, 8, x_17); -lean_ctor_set(x_21, 9, x_10); -lean_ctor_set_uint8(x_21, sizeof(void*)*10, x_20); -x_22 = l_Lean_Elab_Command_instInhabitedScope___closed__2; -x_23 = lean_box(0); -x_24 = l_Lean_Elab_Command_mkState___closed__1; -lean_inc(x_7); -x_25 = lean_alloc_ctor(0, 9, 1); -lean_ctor_set(x_25, 0, x_22); -lean_ctor_set(x_25, 1, x_7); -lean_ctor_set(x_25, 2, x_23); -lean_ctor_set(x_25, 3, x_16); -lean_ctor_set(x_25, 4, x_16); -lean_ctor_set(x_25, 5, x_24); -lean_ctor_set(x_25, 6, x_24); -lean_ctor_set(x_25, 7, x_16); -lean_ctor_set(x_25, 8, x_16); -lean_ctor_set_uint8(x_25, sizeof(void*)*9, x_20); -lean_ctor_set_tag(x_11, 1); -lean_ctor_set(x_11, 1, x_16); -lean_ctor_set(x_11, 0, x_25); -x_26 = l___private_Lean_Elab_Command_0__Lean_Elab_Command_runCore___rarg___closed__4; -x_27 = l_Lean_Elab_Command_mkState___closed__2; -x_28 = l_Lean_Elab_Command_mkState___closed__6; -x_29 = l_Lean_liftCommandElabM___rarg___closed__1; -x_30 = l_Lean_Elab_Command_mkState___closed__11; -lean_inc(x_8); -x_31 = lean_alloc_ctor(0, 8, 0); -lean_ctor_set(x_31, 0, x_15); -lean_ctor_set(x_31, 1, x_26); -lean_ctor_set(x_31, 2, x_11); -lean_ctor_set(x_31, 3, x_27); -lean_ctor_set(x_31, 4, x_8); -lean_ctor_set(x_31, 5, x_28); -lean_ctor_set(x_31, 6, x_29); -lean_ctor_set(x_31, 7, x_30); -x_32 = lean_st_mk_ref(x_31, 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); -lean_inc(x_33); -x_35 = lean_apply_3(x_1, x_21, x_33, x_34); -if (lean_obj_tag(x_35) == 0) -{ -lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; 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_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_33, x_37); -lean_dec(x_33); -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_take(x_3, 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_ctor_get(x_39, 0); -lean_inc(x_44); -x_45 = lean_ctor_get(x_39, 1); -lean_inc(x_45); -x_46 = lean_ctor_get(x_39, 7); -lean_inc(x_46); -lean_dec(x_39); -x_47 = !lean_is_exclusive(x_42); -if (x_47 == 0) -{ -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_42, 3); -x_49 = lean_ctor_get(x_42, 0); -lean_dec(x_49); -x_50 = l_Lean_PersistentArray_append___rarg(x_48, x_46); -lean_dec(x_46); -lean_ctor_set(x_42, 3, x_50); -lean_ctor_set(x_42, 0, x_44); -x_51 = lean_st_ref_set(x_3, x_42, x_43); -x_52 = !lean_is_exclusive(x_51); -if (x_52 == 0) -{ -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; -x_53 = lean_ctor_get(x_51, 1); -x_54 = lean_ctor_get(x_51, 0); -lean_dec(x_54); -x_55 = l_Lean_MessageLog_toArray(x_45); -lean_dec(x_45); -x_56 = lean_array_size(x_55); -x_57 = 0; -x_58 = l_Lean_liftCommandElabM___rarg___closed__2; -x_59 = l_Array_forInUnsafe_loop___at_Lean_liftCommandElabM___spec__1(x_58, x_55, x_56, x_57, x_58); -lean_dec(x_55); -x_60 = lean_ctor_get(x_59, 0); -lean_inc(x_60); -lean_dec(x_59); -if (lean_obj_tag(x_60) == 0) -{ -lean_object* x_61; -x_61 = l_Lean_liftCommandElabM___rarg___closed__4; -if (lean_obj_tag(x_61) == 0) -{ -lean_ctor_set(x_51, 0, x_36); -return x_51; -} -else -{ -lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; -lean_free_object(x_51); -lean_dec(x_36); -x_62 = lean_ctor_get(x_61, 0); -lean_inc(x_62); -x_63 = lean_ctor_get(x_62, 4); -lean_inc(x_63); -lean_dec(x_62); -x_64 = l_Lean_throwError___at_Lean_realizeGlobalConstCore___spec__3(x_63, x_2, x_3, x_53); -x_65 = !lean_is_exclusive(x_64); -if (x_65 == 0) -{ -return x_64; -} -else -{ -lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_66 = lean_ctor_get(x_64, 0); -x_67 = lean_ctor_get(x_64, 1); -lean_inc(x_67); -lean_inc(x_66); -lean_dec(x_64); -x_68 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_68, 0, x_66); -lean_ctor_set(x_68, 1, x_67); -return x_68; -} -} -} -else -{ -lean_object* x_69; -x_69 = lean_ctor_get(x_60, 0); -lean_inc(x_69); -lean_dec(x_60); -if (lean_obj_tag(x_69) == 0) -{ -lean_ctor_set(x_51, 0, x_36); -return x_51; -} -else -{ -lean_object* x_70; lean_object* x_71; lean_object* x_72; uint8_t x_73; -lean_free_object(x_51); -lean_dec(x_36); -x_70 = lean_ctor_get(x_69, 0); -lean_inc(x_70); -lean_dec(x_69); -x_71 = lean_ctor_get(x_70, 4); -lean_inc(x_71); -lean_dec(x_70); -x_72 = l_Lean_throwError___at_Lean_realizeGlobalConstCore___spec__3(x_71, x_2, x_3, x_53); -x_73 = !lean_is_exclusive(x_72); -if (x_73 == 0) -{ -return x_72; -} -else -{ -lean_object* x_74; lean_object* x_75; lean_object* x_76; -x_74 = lean_ctor_get(x_72, 0); -x_75 = lean_ctor_get(x_72, 1); -lean_inc(x_75); -lean_inc(x_74); -lean_dec(x_72); -x_76 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_76, 0, x_74); -lean_ctor_set(x_76, 1, x_75); -return x_76; -} -} +lean_dec(x_5); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, 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; } } else { -lean_object* x_77; lean_object* x_78; size_t x_79; size_t x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; -x_77 = lean_ctor_get(x_51, 1); -lean_inc(x_77); -lean_dec(x_51); -x_78 = l_Lean_MessageLog_toArray(x_45); -lean_dec(x_45); -x_79 = lean_array_size(x_78); -x_80 = 0; -x_81 = l_Lean_liftCommandElabM___rarg___closed__2; -x_82 = l_Array_forInUnsafe_loop___at_Lean_liftCommandElabM___spec__1(x_81, x_78, x_79, x_80, x_81); -lean_dec(x_78); -x_83 = lean_ctor_get(x_82, 0); -lean_inc(x_83); -lean_dec(x_82); -if (lean_obj_tag(x_83) == 0) +uint8_t x_13; +x_13 = !lean_is_exclusive(x_5); +if (x_13 == 0) { -lean_object* x_84; -x_84 = l_Lean_liftCommandElabM___rarg___closed__4; -if (lean_obj_tag(x_84) == 0) +lean_object* x_14; uint8_t x_15; +x_14 = lean_ctor_get(x_5, 0); +x_15 = l_Lean_Exception_isInterrupt(x_14); +if (x_15 == 0) { -lean_object* x_85; -x_85 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_85, 0, x_36); -lean_ctor_set(x_85, 1, x_77); -return x_85; +lean_object* x_16; +x_16 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_16, 0, x_14); +lean_ctor_set_tag(x_5, 0); +lean_ctor_set(x_5, 0, x_16); +return x_5; } 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_dec(x_36); -x_86 = lean_ctor_get(x_84, 0); -lean_inc(x_86); -x_87 = lean_ctor_get(x_86, 4); -lean_inc(x_87); -lean_dec(x_86); -x_88 = l_Lean_throwError___at_Lean_realizeGlobalConstCore___spec__3(x_87, x_2, x_3, x_77); -x_89 = lean_ctor_get(x_88, 0); -lean_inc(x_89); -x_90 = lean_ctor_get(x_88, 1); -lean_inc(x_90); -if (lean_is_exclusive(x_88)) { - lean_ctor_release(x_88, 0); - lean_ctor_release(x_88, 1); - x_91 = x_88; -} else { - lean_dec_ref(x_88); - x_91 = lean_box(0); -} -if (lean_is_scalar(x_91)) { - x_92 = lean_alloc_ctor(1, 2, 0); -} else { - x_92 = x_91; -} -lean_ctor_set(x_92, 0, x_89); -lean_ctor_set(x_92, 1, x_90); -return x_92; +return x_5; } } else { -lean_object* x_93; -x_93 = lean_ctor_get(x_83, 0); -lean_inc(x_93); -lean_dec(x_83); -if (lean_obj_tag(x_93) == 0) -{ -lean_object* x_94; -x_94 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_94, 0, x_36); -lean_ctor_set(x_94, 1, x_77); -return x_94; -} -else +lean_object* x_17; lean_object* x_18; uint8_t x_19; +x_17 = lean_ctor_get(x_5, 0); +x_18 = lean_ctor_get(x_5, 1); +lean_inc(x_18); +lean_inc(x_17); +lean_dec(x_5); +x_19 = l_Lean_Exception_isInterrupt(x_17); +if (x_19 == 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_36); -x_95 = lean_ctor_get(x_93, 0); -lean_inc(x_95); -lean_dec(x_93); -x_96 = lean_ctor_get(x_95, 4); -lean_inc(x_96); -lean_dec(x_95); -x_97 = l_Lean_throwError___at_Lean_realizeGlobalConstCore___spec__3(x_96, x_2, x_3, x_77); -x_98 = lean_ctor_get(x_97, 0); -lean_inc(x_98); -x_99 = lean_ctor_get(x_97, 1); -lean_inc(x_99); -if (lean_is_exclusive(x_97)) { - lean_ctor_release(x_97, 0); - lean_ctor_release(x_97, 1); - x_100 = x_97; -} else { - lean_dec_ref(x_97); - x_100 = lean_box(0); -} -if (lean_is_scalar(x_100)) { - x_101 = lean_alloc_ctor(1, 2, 0); -} else { - x_101 = x_100; -} -lean_ctor_set(x_101, 0, x_98); -lean_ctor_set(x_101, 1, x_99); -return x_101; -} -} -} +lean_object* x_20; lean_object* x_21; +x_20 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_20, 0, x_17); +x_21 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_21, 0, x_20); +lean_ctor_set(x_21, 1, x_18); +return x_21; } else { -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; size_t x_114; size_t x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; -x_102 = lean_ctor_get(x_42, 1); -x_103 = lean_ctor_get(x_42, 2); -x_104 = lean_ctor_get(x_42, 3); -x_105 = lean_ctor_get(x_42, 4); -x_106 = lean_ctor_get(x_42, 5); -x_107 = lean_ctor_get(x_42, 6); -lean_inc(x_107); -lean_inc(x_106); -lean_inc(x_105); -lean_inc(x_104); -lean_inc(x_103); -lean_inc(x_102); -lean_dec(x_42); -x_108 = l_Lean_PersistentArray_append___rarg(x_104, x_46); -lean_dec(x_46); -x_109 = lean_alloc_ctor(0, 7, 0); -lean_ctor_set(x_109, 0, x_44); -lean_ctor_set(x_109, 1, x_102); -lean_ctor_set(x_109, 2, x_103); -lean_ctor_set(x_109, 3, x_108); -lean_ctor_set(x_109, 4, x_105); -lean_ctor_set(x_109, 5, x_106); -lean_ctor_set(x_109, 6, x_107); -x_110 = lean_st_ref_set(x_3, x_109, x_43); -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_110); - x_112 = lean_box(0); -} -x_113 = l_Lean_MessageLog_toArray(x_45); -lean_dec(x_45); -x_114 = lean_array_size(x_113); -x_115 = 0; -x_116 = l_Lean_liftCommandElabM___rarg___closed__2; -x_117 = l_Array_forInUnsafe_loop___at_Lean_liftCommandElabM___spec__1(x_116, x_113, x_114, x_115, x_116); -lean_dec(x_113); -x_118 = lean_ctor_get(x_117, 0); -lean_inc(x_118); -lean_dec(x_117); -if (lean_obj_tag(x_118) == 0) -{ -lean_object* x_119; -x_119 = l_Lean_liftCommandElabM___rarg___closed__4; -if (lean_obj_tag(x_119) == 0) -{ -lean_object* x_120; -if (lean_is_scalar(x_112)) { - x_120 = lean_alloc_ctor(0, 2, 0); -} else { - x_120 = x_112; +lean_object* x_22; +x_22 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_22, 0, x_17); +lean_ctor_set(x_22, 1, x_18); +return x_22; } -lean_ctor_set(x_120, 0, x_36); -lean_ctor_set(x_120, 1, x_111); -return x_120; } -else -{ -lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; -lean_dec(x_112); -lean_dec(x_36); -x_121 = lean_ctor_get(x_119, 0); -lean_inc(x_121); -x_122 = lean_ctor_get(x_121, 4); -lean_inc(x_122); -lean_dec(x_121); -x_123 = l_Lean_throwError___at_Lean_realizeGlobalConstCore___spec__3(x_122, x_2, x_3, x_111); -x_124 = lean_ctor_get(x_123, 0); -lean_inc(x_124); -x_125 = lean_ctor_get(x_123, 1); -lean_inc(x_125); -if (lean_is_exclusive(x_123)) { - lean_ctor_release(x_123, 0); - lean_ctor_release(x_123, 1); - x_126 = x_123; -} else { - lean_dec_ref(x_123); - x_126 = lean_box(0); } -if (lean_is_scalar(x_126)) { - x_127 = lean_alloc_ctor(1, 2, 0); -} else { - x_127 = x_126; } -lean_ctor_set(x_127, 0, x_124); -lean_ctor_set(x_127, 1, x_125); -return x_127; } +LEAN_EXPORT lean_object* l_Lean_liftCommandElabM___rarg(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; +x_6 = lean_alloc_closure((void*)(l_Lean_liftCommandElabM___rarg___lambda__1), 4, 1); +lean_closure_set(x_6, 0, x_1); +x_7 = l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg(x_6, x_2, x_3, x_4, x_5); +if (lean_obj_tag(x_7) == 0) +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; +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_MonadExcept_ofExcept___at_Lean_liftCommandElabM___spec__1___rarg(x_8, x_3, x_4, x_9); +lean_dec(x_8); +return x_10; } else { -lean_object* x_128; -x_128 = lean_ctor_get(x_118, 0); -lean_inc(x_128); -lean_dec(x_118); -if (lean_obj_tag(x_128) == 0) +uint8_t x_11; +x_11 = !lean_is_exclusive(x_7); +if (x_11 == 0) { -lean_object* x_129; -if (lean_is_scalar(x_112)) { - x_129 = lean_alloc_ctor(0, 2, 0); -} else { - x_129 = x_112; -} -lean_ctor_set(x_129, 0, x_36); -lean_ctor_set(x_129, 1, x_111); -return x_129; +return x_7; } 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; lean_object* x_136; -lean_dec(x_112); -lean_dec(x_36); -x_130 = lean_ctor_get(x_128, 0); -lean_inc(x_130); -lean_dec(x_128); -x_131 = lean_ctor_get(x_130, 4); -lean_inc(x_131); -lean_dec(x_130); -x_132 = l_Lean_throwError___at_Lean_realizeGlobalConstCore___spec__3(x_131, x_2, x_3, x_111); -x_133 = lean_ctor_get(x_132, 0); -lean_inc(x_133); -x_134 = lean_ctor_get(x_132, 1); -lean_inc(x_134); -if (lean_is_exclusive(x_132)) { - lean_ctor_release(x_132, 0); - lean_ctor_release(x_132, 1); - x_135 = x_132; -} else { - lean_dec_ref(x_132); - x_135 = lean_box(0); +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_7, 0); +x_13 = lean_ctor_get(x_7, 1); +lean_inc(x_13); +lean_inc(x_12); +lean_dec(x_7); +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; } -if (lean_is_scalar(x_135)) { - x_136 = lean_alloc_ctor(1, 2, 0); -} else { - x_136 = x_135; } -lean_ctor_set(x_136, 0, x_133); -lean_ctor_set(x_136, 1, x_134); -return x_136; } } +LEAN_EXPORT lean_object* l_Lean_liftCommandElabM(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_liftCommandElabM___rarg___boxed), 5, 0); +return x_2; } } -else -{ -uint8_t x_137; -lean_dec(x_33); -x_137 = !lean_is_exclusive(x_35); -if (x_137 == 0) +LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_liftCommandElabM___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: { -return x_35; +lean_object* x_5; +x_5 = l_MonadExcept_ofExcept___at_Lean_liftCommandElabM___spec__1___rarg(x_1, x_2, x_3, x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_5; } -else -{ -lean_object* x_138; lean_object* x_139; lean_object* x_140; -x_138 = lean_ctor_get(x_35, 0); -x_139 = lean_ctor_get(x_35, 1); -lean_inc(x_139); -lean_inc(x_138); -lean_dec(x_35); -x_140 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_140, 0, x_138); -lean_ctor_set(x_140, 1, x_139); -return x_140; } +LEAN_EXPORT lean_object* l_Lean_liftCommandElabM___rarg___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_liftCommandElabM___rarg(x_1, x_6, x_3, x_4, x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_7; } } -else +LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoTree___at_Lean_withSetOptionIn___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: { -lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; uint8_t x_148; 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_141 = lean_ctor_get(x_11, 0); -x_142 = lean_ctor_get(x_11, 1); -lean_inc(x_142); -lean_inc(x_141); -lean_dec(x_11); -x_143 = lean_ctor_get(x_141, 0); -lean_inc(x_143); -lean_dec(x_141); -x_144 = lean_box(0); -x_145 = lean_box(0); -x_146 = lean_unsigned_to_nat(0u); -x_147 = l_Lean_firstFrontendMacroScope; -x_148 = 0; -lean_inc(x_10); -lean_inc(x_9); +lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; +x_5 = lean_st_ref_get(x_3, x_4); +x_6 = lean_ctor_get(x_5, 0); lean_inc(x_6); -lean_inc(x_5); -x_149 = lean_alloc_ctor(0, 10, 1); -lean_ctor_set(x_149, 0, x_5); -lean_ctor_set(x_149, 1, x_6); -lean_ctor_set(x_149, 2, x_146); -lean_ctor_set(x_149, 3, x_146); -lean_ctor_set(x_149, 4, x_144); -lean_ctor_set(x_149, 5, x_147); -lean_ctor_set(x_149, 6, x_9); -lean_ctor_set(x_149, 7, x_145); -lean_ctor_set(x_149, 8, x_145); -lean_ctor_set(x_149, 9, x_10); -lean_ctor_set_uint8(x_149, sizeof(void*)*10, x_148); -x_150 = l_Lean_Elab_Command_instInhabitedScope___closed__2; -x_151 = lean_box(0); -x_152 = l_Lean_Elab_Command_mkState___closed__1; +x_7 = lean_ctor_get(x_6, 6); lean_inc(x_7); -x_153 = lean_alloc_ctor(0, 9, 1); -lean_ctor_set(x_153, 0, x_150); -lean_ctor_set(x_153, 1, x_7); -lean_ctor_set(x_153, 2, x_151); -lean_ctor_set(x_153, 3, x_144); -lean_ctor_set(x_153, 4, x_144); -lean_ctor_set(x_153, 5, x_152); -lean_ctor_set(x_153, 6, x_152); -lean_ctor_set(x_153, 7, x_144); -lean_ctor_set(x_153, 8, x_144); -lean_ctor_set_uint8(x_153, sizeof(void*)*9, x_148); -x_154 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_154, 0, x_153); -lean_ctor_set(x_154, 1, x_144); -x_155 = l___private_Lean_Elab_Command_0__Lean_Elab_Command_runCore___rarg___closed__4; -x_156 = l_Lean_Elab_Command_mkState___closed__2; -x_157 = l_Lean_Elab_Command_mkState___closed__6; -x_158 = l_Lean_liftCommandElabM___rarg___closed__1; -x_159 = l_Lean_Elab_Command_mkState___closed__11; -lean_inc(x_8); -x_160 = lean_alloc_ctor(0, 8, 0); -lean_ctor_set(x_160, 0, x_143); -lean_ctor_set(x_160, 1, x_155); -lean_ctor_set(x_160, 2, x_154); -lean_ctor_set(x_160, 3, x_156); -lean_ctor_set(x_160, 4, x_8); -lean_ctor_set(x_160, 5, x_157); -lean_ctor_set(x_160, 6, x_158); -lean_ctor_set(x_160, 7, x_159); -x_161 = lean_st_mk_ref(x_160, x_142); -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_inc(x_162); -x_164 = lean_apply_3(x_1, x_149, x_162, x_163); -if (lean_obj_tag(x_164) == 0) +lean_dec(x_6); +x_8 = lean_ctor_get_uint8(x_7, sizeof(void*)*2); +lean_dec(x_7); +if (x_8 == 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; lean_object* x_188; size_t x_189; size_t x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; -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_162, x_166); -lean_dec(x_162); -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 = lean_st_ref_take(x_3, x_169); -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_168, 0); -lean_inc(x_173); -x_174 = lean_ctor_get(x_168, 1); -lean_inc(x_174); -x_175 = lean_ctor_get(x_168, 7); -lean_inc(x_175); -lean_dec(x_168); -x_176 = lean_ctor_get(x_171, 1); -lean_inc(x_176); -x_177 = lean_ctor_get(x_171, 2); -lean_inc(x_177); -x_178 = lean_ctor_get(x_171, 3); -lean_inc(x_178); -x_179 = lean_ctor_get(x_171, 4); -lean_inc(x_179); -x_180 = lean_ctor_get(x_171, 5); -lean_inc(x_180); -x_181 = lean_ctor_get(x_171, 6); -lean_inc(x_181); -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); - lean_ctor_release(x_171, 6); - x_182 = x_171; -} else { - lean_dec_ref(x_171); - x_182 = lean_box(0); +uint8_t x_9; +lean_dec(x_1); +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); +lean_dec(x_10); +x_11 = lean_box(0); +lean_ctor_set(x_5, 0, x_11); +return x_5; } -x_183 = l_Lean_PersistentArray_append___rarg(x_178, x_175); -lean_dec(x_175); -if (lean_is_scalar(x_182)) { - x_184 = lean_alloc_ctor(0, 7, 0); -} else { - x_184 = x_182; -} -lean_ctor_set(x_184, 0, x_173); -lean_ctor_set(x_184, 1, x_176); -lean_ctor_set(x_184, 2, x_177); -lean_ctor_set(x_184, 3, x_183); -lean_ctor_set(x_184, 4, x_179); -lean_ctor_set(x_184, 5, x_180); -lean_ctor_set(x_184, 6, x_181); -x_185 = lean_st_ref_set(x_3, x_184, x_172); -x_186 = lean_ctor_get(x_185, 1); -lean_inc(x_186); -if (lean_is_exclusive(x_185)) { - lean_ctor_release(x_185, 0); - lean_ctor_release(x_185, 1); - x_187 = x_185; -} else { - lean_dec_ref(x_185); - x_187 = lean_box(0); +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_5, 1); +lean_inc(x_12); +lean_dec(x_5); +x_13 = lean_box(0); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_13); +lean_ctor_set(x_14, 1, x_12); +return x_14; } -x_188 = l_Lean_MessageLog_toArray(x_174); -lean_dec(x_174); -x_189 = lean_array_size(x_188); -x_190 = 0; -x_191 = l_Lean_liftCommandElabM___rarg___closed__2; -x_192 = l_Array_forInUnsafe_loop___at_Lean_liftCommandElabM___spec__1(x_191, x_188, x_189, x_190, x_191); -lean_dec(x_188); -x_193 = lean_ctor_get(x_192, 0); -lean_inc(x_193); -lean_dec(x_192); -if (lean_obj_tag(x_193) == 0) +} +else { -lean_object* x_194; -x_194 = l_Lean_liftCommandElabM___rarg___closed__4; -if (lean_obj_tag(x_194) == 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; +x_15 = lean_ctor_get(x_5, 1); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_st_ref_take(x_3, x_15); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_17, 6); +lean_inc(x_18); +x_19 = lean_ctor_get(x_16, 1); +lean_inc(x_19); +lean_dec(x_16); +x_20 = !lean_is_exclusive(x_17); +if (x_20 == 0) { -lean_object* x_195; -if (lean_is_scalar(x_187)) { - x_195 = lean_alloc_ctor(0, 2, 0); -} else { - x_195 = x_187; +lean_object* x_21; uint8_t x_22; +x_21 = lean_ctor_get(x_17, 6); +lean_dec(x_21); +x_22 = !lean_is_exclusive(x_18); +if (x_22 == 0) +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; +x_23 = lean_ctor_get(x_18, 1); +x_24 = l_Lean_PersistentArray_push___rarg(x_23, x_1); +lean_ctor_set(x_18, 1, x_24); +x_25 = lean_st_ref_set(x_3, x_17, x_19); +x_26 = !lean_is_exclusive(x_25); +if (x_26 == 0) +{ +lean_object* x_27; lean_object* x_28; +x_27 = lean_ctor_get(x_25, 0); +lean_dec(x_27); +x_28 = lean_box(0); +lean_ctor_set(x_25, 0, x_28); +return x_25; +} +else +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_25, 1); +lean_inc(x_29); +lean_dec(x_25); +x_30 = lean_box(0); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_30); +lean_ctor_set(x_31, 1, x_29); +return x_31; } -lean_ctor_set(x_195, 0, x_165); -lean_ctor_set(x_195, 1, x_186); -return x_195; } else { -lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; -lean_dec(x_187); -lean_dec(x_165); -x_196 = lean_ctor_get(x_194, 0); -lean_inc(x_196); -x_197 = lean_ctor_get(x_196, 4); -lean_inc(x_197); -lean_dec(x_196); -x_198 = l_Lean_throwError___at_Lean_realizeGlobalConstCore___spec__3(x_197, x_2, x_3, x_186); -x_199 = lean_ctor_get(x_198, 0); -lean_inc(x_199); -x_200 = lean_ctor_get(x_198, 1); -lean_inc(x_200); -if (lean_is_exclusive(x_198)) { - lean_ctor_release(x_198, 0); - lean_ctor_release(x_198, 1); - x_201 = x_198; +uint8_t x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_32 = lean_ctor_get_uint8(x_18, sizeof(void*)*2); +x_33 = lean_ctor_get(x_18, 0); +x_34 = lean_ctor_get(x_18, 1); +lean_inc(x_34); +lean_inc(x_33); +lean_dec(x_18); +x_35 = l_Lean_PersistentArray_push___rarg(x_34, x_1); +x_36 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_36, 0, x_33); +lean_ctor_set(x_36, 1, x_35); +lean_ctor_set_uint8(x_36, sizeof(void*)*2, x_32); +lean_ctor_set(x_17, 6, x_36); +x_37 = lean_st_ref_set(x_3, x_17, x_19); +x_38 = lean_ctor_get(x_37, 1); +lean_inc(x_38); +if (lean_is_exclusive(x_37)) { + lean_ctor_release(x_37, 0); + lean_ctor_release(x_37, 1); + x_39 = x_37; } else { - lean_dec_ref(x_198); - x_201 = lean_box(0); + lean_dec_ref(x_37); + x_39 = lean_box(0); } -if (lean_is_scalar(x_201)) { - x_202 = lean_alloc_ctor(1, 2, 0); +x_40 = lean_box(0); +if (lean_is_scalar(x_39)) { + x_41 = lean_alloc_ctor(0, 2, 0); } else { - x_202 = x_201; + x_41 = x_39; } -lean_ctor_set(x_202, 0, x_199); -lean_ctor_set(x_202, 1, x_200); -return x_202; +lean_ctor_set(x_41, 0, x_40); +lean_ctor_set(x_41, 1, x_38); +return x_41; } } else { -lean_object* x_203; -x_203 = lean_ctor_get(x_193, 0); -lean_inc(x_203); -lean_dec(x_193); -if (lean_obj_tag(x_203) == 0) -{ -lean_object* x_204; -if (lean_is_scalar(x_187)) { - x_204 = lean_alloc_ctor(0, 2, 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; uint8_t x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; +x_42 = lean_ctor_get(x_17, 0); +x_43 = lean_ctor_get(x_17, 1); +x_44 = lean_ctor_get(x_17, 2); +x_45 = lean_ctor_get(x_17, 3); +x_46 = lean_ctor_get(x_17, 4); +x_47 = lean_ctor_get(x_17, 5); +x_48 = lean_ctor_get(x_17, 7); +lean_inc(x_48); +lean_inc(x_47); +lean_inc(x_46); +lean_inc(x_45); +lean_inc(x_44); +lean_inc(x_43); +lean_inc(x_42); +lean_dec(x_17); +x_49 = lean_ctor_get_uint8(x_18, sizeof(void*)*2); +x_50 = lean_ctor_get(x_18, 0); +lean_inc(x_50); +x_51 = lean_ctor_get(x_18, 1); +lean_inc(x_51); +if (lean_is_exclusive(x_18)) { + lean_ctor_release(x_18, 0); + lean_ctor_release(x_18, 1); + x_52 = x_18; } else { - x_204 = x_187; + lean_dec_ref(x_18); + x_52 = lean_box(0); } -lean_ctor_set(x_204, 0, x_165); -lean_ctor_set(x_204, 1, x_186); -return x_204; +x_53 = l_Lean_PersistentArray_push___rarg(x_51, x_1); +if (lean_is_scalar(x_52)) { + x_54 = lean_alloc_ctor(0, 2, 1); +} else { + x_54 = x_52; } -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_dec(x_187); -lean_dec(x_165); -x_205 = lean_ctor_get(x_203, 0); -lean_inc(x_205); -lean_dec(x_203); -x_206 = lean_ctor_get(x_205, 4); -lean_inc(x_206); -lean_dec(x_205); -x_207 = l_Lean_throwError___at_Lean_realizeGlobalConstCore___spec__3(x_206, x_2, x_3, x_186); -x_208 = lean_ctor_get(x_207, 0); -lean_inc(x_208); -x_209 = lean_ctor_get(x_207, 1); -lean_inc(x_209); -if (lean_is_exclusive(x_207)) { - lean_ctor_release(x_207, 0); - lean_ctor_release(x_207, 1); - x_210 = x_207; +lean_ctor_set(x_54, 0, x_50); +lean_ctor_set(x_54, 1, x_53); +lean_ctor_set_uint8(x_54, sizeof(void*)*2, x_49); +x_55 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_55, 0, x_42); +lean_ctor_set(x_55, 1, x_43); +lean_ctor_set(x_55, 2, x_44); +lean_ctor_set(x_55, 3, x_45); +lean_ctor_set(x_55, 4, x_46); +lean_ctor_set(x_55, 5, x_47); +lean_ctor_set(x_55, 6, x_54); +lean_ctor_set(x_55, 7, x_48); +x_56 = lean_st_ref_set(x_3, x_55, x_19); +x_57 = lean_ctor_get(x_56, 1); +lean_inc(x_57); +if (lean_is_exclusive(x_56)) { + lean_ctor_release(x_56, 0); + lean_ctor_release(x_56, 1); + x_58 = x_56; } else { - lean_dec_ref(x_207); - x_210 = lean_box(0); + lean_dec_ref(x_56); + x_58 = lean_box(0); } -if (lean_is_scalar(x_210)) { - x_211 = lean_alloc_ctor(1, 2, 0); +x_59 = lean_box(0); +if (lean_is_scalar(x_58)) { + x_60 = lean_alloc_ctor(0, 2, 0); } else { - x_211 = x_210; + x_60 = x_58; } -lean_ctor_set(x_211, 0, x_208); -lean_ctor_set(x_211, 1, x_209); -return x_211; +lean_ctor_set(x_60, 0, x_59); +lean_ctor_set(x_60, 1, x_57); +return x_60; } } } -else +} +LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoLeaf___at_Lean_withSetOptionIn___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: { -lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; -lean_dec(x_162); -x_212 = lean_ctor_get(x_164, 0); -lean_inc(x_212); -x_213 = lean_ctor_get(x_164, 1); -lean_inc(x_213); -if (lean_is_exclusive(x_164)) { - lean_ctor_release(x_164, 0); - lean_ctor_release(x_164, 1); - x_214 = x_164; -} else { - lean_dec_ref(x_164); - x_214 = lean_box(0); +lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; +x_5 = lean_st_ref_get(x_3, x_4); +x_6 = lean_ctor_get(x_5, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_6, 6); +lean_inc(x_7); +lean_dec(x_6); +x_8 = lean_ctor_get_uint8(x_7, sizeof(void*)*2); +lean_dec(x_7); +if (x_8 == 0) +{ +uint8_t x_9; +lean_dec(x_1); +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); +lean_dec(x_10); +x_11 = lean_box(0); +lean_ctor_set(x_5, 0, x_11); +return x_5; } -if (lean_is_scalar(x_214)) { - x_215 = lean_alloc_ctor(1, 2, 0); -} else { - x_215 = x_214; +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_5, 1); +lean_inc(x_12); +lean_dec(x_5); +x_13 = lean_box(0); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_13); +lean_ctor_set(x_14, 1, x_12); +return x_14; } -lean_ctor_set(x_215, 0, x_212); -lean_ctor_set(x_215, 1, x_213); -return x_215; } +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_15 = lean_ctor_get(x_5, 1); +lean_inc(x_15); +lean_dec(x_5); +x_16 = l_Lean_Elab_Command_mkState___closed__11; +x_17 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_17, 0, x_1); +lean_ctor_set(x_17, 1, x_16); +x_18 = l_Lean_Elab_pushInfoTree___at_Lean_withSetOptionIn___spec__4(x_17, x_2, x_3, x_15); +return x_18; } } } -LEAN_EXPORT lean_object* l_Lean_liftCommandElabM(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_addCompletionInfo___at_Lean_withSetOptionIn___spec__2(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_liftCommandElabM___rarg___boxed), 4, 0); -return x_2; +lean_object* x_5; lean_object* x_6; +x_5 = lean_alloc_ctor(6, 1, 0); +lean_ctor_set(x_5, 0, x_1); +x_6 = l_Lean_Elab_pushInfoLeaf___at_Lean_withSetOptionIn___spec__3(x_5, x_2, x_3, x_4); +return x_6; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_liftCommandElabM___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_withSetOptionIn___spec__5(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_liftCommandElabM___spec__1(x_1, x_2, x_6, x_7, x_5); +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_5 = l_Lean_Elab_Command_getRef(x_2, x_3, x_4); +x_6 = lean_ctor_get(x_5, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_5, 1); +lean_inc(x_7); lean_dec(x_5); +x_8 = lean_ctor_get(x_2, 4); +lean_inc(x_8); +lean_inc(x_8); +x_9 = l_Lean_Elab_getBetterRef(x_6, x_8); +lean_dec(x_6); +x_10 = l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1(x_1, x_2, x_3, x_7); +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_12 = lean_ctor_get(x_10, 0); +x_13 = lean_ctor_get(x_10, 1); +x_14 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_12, x_8, x_2, x_3, x_13); lean_dec(x_2); -lean_dec(x_1); -return x_8; -} +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 0) +{ +lean_object* x_16; +x_16 = lean_ctor_get(x_14, 0); +lean_ctor_set(x_10, 1, x_16); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set_tag(x_14, 1); +lean_ctor_set(x_14, 0, x_10); +return x_14; } -LEAN_EXPORT lean_object* l_Lean_liftCommandElabM___rarg___lambda__1___boxed(lean_object* x_1) { -_start: +else { -lean_object* x_2; -x_2 = l_Lean_liftCommandElabM___rarg___lambda__1(x_1); -lean_dec(x_1); -return x_2; +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_14, 0); +x_18 = lean_ctor_get(x_14, 1); +lean_inc(x_18); +lean_inc(x_17); +lean_dec(x_14); +lean_ctor_set(x_10, 1, x_17); +lean_ctor_set(x_10, 0, x_9); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_10); +lean_ctor_set(x_19, 1, x_18); +return x_19; } } -LEAN_EXPORT lean_object* l_Lean_liftCommandElabM___rarg___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_liftCommandElabM___rarg(x_1, x_2, x_3, x_4); -lean_dec(x_3); +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_20 = lean_ctor_get(x_10, 0); +x_21 = lean_ctor_get(x_10, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_10); +x_22 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_20, x_8, x_2, x_3, x_21); lean_dec(x_2); -return x_5; +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +if (lean_is_exclusive(x_22)) { + lean_ctor_release(x_22, 0); + lean_ctor_release(x_22, 1); + x_25 = x_22; +} else { + lean_dec_ref(x_22); + x_25 = lean_box(0); } +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_9); +lean_ctor_set(x_26, 1, x_23); +if (lean_is_scalar(x_25)) { + x_27 = lean_alloc_ctor(1, 2, 0); +} else { + x_27 = x_25; + lean_ctor_set_tag(x_27, 1); } -LEAN_EXPORT lean_object* l_Lean_Elab_addCompletionInfo___at_Lean_withSetOptionIn___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -lean_object* x_5; lean_object* x_6; -x_5 = lean_alloc_ctor(6, 1, 0); -lean_ctor_set(x_5, 0, x_1); -x_6 = l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_expandDeclId___spec__11(x_5, x_2, x_3, x_4); -return x_6; +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_24); +return x_27; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_withSetOptionIn___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +} +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_withSetOptionIn___spec__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; lean_object* x_9; lean_object* x_10; uint8_t x_11; @@ -40591,7 +37153,7 @@ return x_27; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___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_EXPORT lean_object* l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; uint8_t x_8; @@ -40639,7 +37201,7 @@ return x_22; } } } -static lean_object* _init_l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__4___closed__1() { +static lean_object* _init_l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6___closed__1() { _start: { lean_object* x_1; @@ -40647,16 +37209,16 @@ x_1 = lean_mk_string_unchecked("type mismatch at set_option", 27, 27); return x_1; } } -static lean_object* _init_l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__4___closed__2() { +static lean_object* _init_l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__4___closed__1; +x_1 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___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_EXPORT lean_object* l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___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: { lean_object* x_7; uint8_t x_8; @@ -40667,8 +37229,8 @@ if (x_8 == 0) lean_object* x_9; lean_object* x_10; uint8_t x_11; lean_dec(x_3); lean_dec(x_1); -x_9 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__4___closed__2; -x_10 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_9, x_4, x_5, x_6); +x_9 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6___closed__2; +x_10 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__7(x_9, x_4, x_5, x_6); x_11 = !lean_is_exclusive(x_10); if (x_11 == 0) { @@ -40692,7 +37254,7 @@ else { lean_object* x_15; lean_object* x_16; x_15 = lean_box(0); -x_16 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__4___lambda__1(x_1, x_3, x_15, x_4, x_5, x_6); +x_16 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6___lambda__1(x_1, x_3, x_15, x_4, x_5, x_6); lean_dec(x_4); return x_16; } @@ -40801,7 +37363,7 @@ lean_ctor_set(x_26, 1, x_21); lean_ctor_set(x_26, 2, x_25); x_27 = lean_alloc_ctor(4, 1, 0); lean_ctor_set(x_27, 0, x_26); -x_28 = l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_expandDeclId___spec__11(x_27, x_3, x_4, x_24); +x_28 = l_Lean_Elab_pushInfoLeaf___at_Lean_withSetOptionIn___spec__3(x_27, x_3, x_4, x_24); x_29 = !lean_is_exclusive(x_28); if (x_29 == 0) { @@ -40853,7 +37415,7 @@ x_44 = l_Lean_Elab_logException___at_Lean_Elab_Command_runLinters___spec__1___cl lean_ctor_set_tag(x_28, 7); lean_ctor_set(x_28, 1, x_44); lean_ctor_set(x_28, 0, x_2); -x_45 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__3(x_28, x_3, x_4, x_30); +x_45 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__5(x_28, x_3, x_4, x_30); return x_45; } else @@ -40868,7 +37430,7 @@ x_48 = l_Lean_Elab_logException___at_Lean_Elab_Command_runLinters___spec__1___cl lean_ctor_set_tag(x_28, 7); lean_ctor_set(x_28, 1, x_48); lean_ctor_set(x_28, 0, x_47); -x_49 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__3(x_28, x_3, x_4, x_30); +x_49 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__5(x_28, x_3, x_4, x_30); return x_49; } } @@ -40878,7 +37440,7 @@ lean_object* x_50; lean_object* x_51; lean_free_object(x_28); lean_dec(x_2); x_50 = l_Lean_Elab_elabSetOption___at_Lean_withSetOptionIn___spec__1___closed__5; -x_51 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__4(x_21, x_23, x_50, x_3, x_4, x_30); +x_51 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6(x_21, x_23, x_50, x_3, x_4, x_30); lean_dec(x_23); return x_51; } @@ -40890,7 +37452,7 @@ lean_dec(x_34); lean_free_object(x_28); lean_dec(x_2); x_52 = l_Lean_Elab_elabSetOption___at_Lean_withSetOptionIn___spec__1___closed__6; -x_53 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__4(x_21, x_23, x_52, x_3, x_4, x_30); +x_53 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6(x_21, x_23, x_52, x_3, x_4, x_30); lean_dec(x_23); return x_53; } @@ -40909,7 +37471,7 @@ x_56 = l_Lean_Elab_logException___at_Lean_Elab_Command_runLinters___spec__1___cl lean_ctor_set_tag(x_16, 7); lean_ctor_set(x_16, 1, x_56); lean_ctor_set(x_16, 0, x_28); -x_57 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__3(x_16, x_3, x_4, x_30); +x_57 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__5(x_16, x_3, x_4, x_30); return x_57; } } @@ -40924,7 +37486,7 @@ if (x_58 == 0) { lean_object* x_59; lean_ctor_set_tag(x_33, 3); -x_59 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__4(x_21, x_23, x_33, x_3, x_4, x_30); +x_59 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6(x_21, x_23, x_33, x_3, x_4, x_30); lean_dec(x_23); return x_59; } @@ -40936,7 +37498,7 @@ lean_inc(x_60); lean_dec(x_33); x_61 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_61, 0, x_60); -x_62 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__4(x_21, x_23, x_61, x_3, x_4, x_30); +x_62 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6(x_21, x_23, x_61, x_3, x_4, x_30); lean_dec(x_23); return x_62; } @@ -40953,7 +37515,7 @@ if (x_63 == 0) { lean_object* x_64; lean_ctor_set_tag(x_32, 0); -x_64 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__4(x_21, x_23, x_32, x_3, x_4, x_30); +x_64 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6(x_21, x_23, x_32, x_3, x_4, x_30); lean_dec(x_23); return x_64; } @@ -40965,7 +37527,7 @@ lean_inc(x_65); lean_dec(x_32); x_66 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_66, 0, x_65); -x_67 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__4(x_21, x_23, x_66, x_3, x_4, x_30); +x_67 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6(x_21, x_23, x_66, x_3, x_4, x_30); lean_dec(x_23); return x_67; } @@ -41026,7 +37588,7 @@ x_80 = l_Lean_Elab_logException___at_Lean_Elab_Command_runLinters___spec__1___cl x_81 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_81, 0, x_79); lean_ctor_set(x_81, 1, x_80); -x_82 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__3(x_81, x_3, x_4, x_68); +x_82 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__5(x_81, x_3, x_4, x_68); return x_82; } else @@ -41034,7 +37596,7 @@ else lean_object* x_83; lean_object* x_84; lean_dec(x_2); x_83 = l_Lean_Elab_elabSetOption___at_Lean_withSetOptionIn___spec__1___closed__5; -x_84 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__4(x_21, x_23, x_83, x_3, x_4, x_68); +x_84 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6(x_21, x_23, x_83, x_3, x_4, x_68); lean_dec(x_23); return x_84; } @@ -41045,7 +37607,7 @@ lean_object* x_85; lean_object* x_86; lean_dec(x_71); lean_dec(x_2); x_85 = l_Lean_Elab_elabSetOption___at_Lean_withSetOptionIn___spec__1___closed__6; -x_86 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__4(x_21, x_23, x_85, x_3, x_4, x_68); +x_86 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6(x_21, x_23, x_85, x_3, x_4, x_68); lean_dec(x_23); return x_86; } @@ -41064,7 +37626,7 @@ x_90 = l_Lean_Elab_logException___at_Lean_Elab_Command_runLinters___spec__1___cl lean_ctor_set_tag(x_16, 7); lean_ctor_set(x_16, 1, x_90); lean_ctor_set(x_16, 0, x_89); -x_91 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__3(x_16, x_3, x_4, x_68); +x_91 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__5(x_16, x_3, x_4, x_68); return x_91; } } @@ -41089,7 +37651,7 @@ if (lean_is_scalar(x_93)) { lean_ctor_set_tag(x_94, 3); } lean_ctor_set(x_94, 0, x_92); -x_95 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__4(x_21, x_23, x_94, x_3, x_4, x_68); +x_95 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6(x_21, x_23, x_94, x_3, x_4, x_68); lean_dec(x_23); return x_95; } @@ -41115,7 +37677,7 @@ if (lean_is_scalar(x_97)) { lean_ctor_set_tag(x_98, 0); } lean_ctor_set(x_98, 0, x_96); -x_99 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__4(x_21, x_23, x_98, x_3, x_4, x_68); +x_99 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6(x_21, x_23, x_98, x_3, x_4, x_68); lean_dec(x_23); return x_99; } @@ -41191,7 +37753,7 @@ lean_ctor_set(x_118, 1, x_113); lean_ctor_set(x_118, 2, x_117); x_119 = lean_alloc_ctor(4, 1, 0); lean_ctor_set(x_119, 0, x_118); -x_120 = l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_expandDeclId___spec__11(x_119, x_3, x_4, x_116); +x_120 = l_Lean_Elab_pushInfoLeaf___at_Lean_withSetOptionIn___spec__3(x_119, x_3, x_4, x_116); x_121 = lean_ctor_get(x_120, 1); lean_inc(x_121); if (lean_is_exclusive(x_120)) { @@ -41255,7 +37817,7 @@ if (lean_is_scalar(x_122)) { } lean_ctor_set(x_135, 0, x_133); lean_ctor_set(x_135, 1, x_134); -x_136 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__3(x_135, x_3, x_4, x_121); +x_136 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__5(x_135, x_3, x_4, x_121); return x_136; } else @@ -41264,7 +37826,7 @@ lean_object* x_137; lean_object* x_138; lean_dec(x_122); lean_dec(x_2); x_137 = l_Lean_Elab_elabSetOption___at_Lean_withSetOptionIn___spec__1___closed__5; -x_138 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__4(x_113, x_115, x_137, x_3, x_4, x_121); +x_138 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6(x_113, x_115, x_137, x_3, x_4, x_121); lean_dec(x_115); return x_138; } @@ -41276,7 +37838,7 @@ lean_dec(x_125); lean_dec(x_122); lean_dec(x_2); x_139 = l_Lean_Elab_elabSetOption___at_Lean_withSetOptionIn___spec__1___closed__6; -x_140 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__4(x_113, x_115, x_139, x_3, x_4, x_121); +x_140 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6(x_113, x_115, x_139, x_3, x_4, x_121); lean_dec(x_115); return x_140; } @@ -41300,7 +37862,7 @@ x_144 = l_Lean_Elab_logException___at_Lean_Elab_Command_runLinters___spec__1___c x_145 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_145, 0, x_143); lean_ctor_set(x_145, 1, x_144); -x_146 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__3(x_145, x_3, x_4, x_121); +x_146 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__5(x_145, x_3, x_4, x_121); return x_146; } } @@ -41325,7 +37887,7 @@ if (lean_is_scalar(x_148)) { lean_ctor_set_tag(x_149, 3); } lean_ctor_set(x_149, 0, x_147); -x_150 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__4(x_113, x_115, x_149, x_3, x_4, x_121); +x_150 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6(x_113, x_115, x_149, x_3, x_4, x_121); lean_dec(x_115); return x_150; } @@ -41351,7 +37913,7 @@ if (lean_is_scalar(x_152)) { lean_ctor_set_tag(x_153, 0); } lean_ctor_set(x_153, 0, x_151); -x_154 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__4(x_113, x_115, x_153, x_3, x_4, x_121); +x_154 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6(x_113, x_115, x_153, x_3, x_4, x_121); lean_dec(x_115); return x_154; } @@ -41574,6 +38136,26 @@ return x_31; } } } +LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoTree___at_Lean_withSetOptionIn___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Lean_Elab_pushInfoTree___at_Lean_withSetOptionIn___spec__4(x_1, x_2, x_3, x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoLeaf___at_Lean_withSetOptionIn___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Lean_Elab_pushInfoLeaf___at_Lean_withSetOptionIn___spec__3(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_addCompletionInfo___at_Lean_withSetOptionIn___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { @@ -41584,31 +38166,40 @@ lean_dec(x_2); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_withSetOptionIn___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_withSetOptionIn___spec__5___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_withSetOptionIn___spec__5(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_withSetOptionIn___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_Lean_throwError___at_Lean_withSetOptionIn___spec__3(x_1, x_2, x_3, x_4); +x_5 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__7(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___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_EXPORT lean_object* l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; -x_7 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__4___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___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_EXPORT lean_object* l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___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) { _start: { lean_object* x_7; -x_7 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__4(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_5); lean_dec(x_2); return x_7; @@ -42232,80 +38823,16 @@ l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_addUnivLeve lean_mark_persistent(l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_addUnivLevel___spec__1___closed__3); l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_addUnivLevel___spec__1___closed__4 = _init_l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_addUnivLevel___spec__1___closed__4(); lean_mark_persistent(l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_addUnivLevel___spec__1___closed__4); -l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__1); -l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__2 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__2(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__2); -l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__3 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__3(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__3); -l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__4 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__4(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__4); -l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__5 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__5(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__5); -l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__6 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__6(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__6); -l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__7 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__7(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__7); -l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__8 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__8(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__8); -l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9___closed__1 = _init_l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9___closed__1(); -lean_mark_persistent(l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9___closed__1); -l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9___closed__2 = _init_l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9___closed__2(); -lean_mark_persistent(l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9___closed__2); -l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__1___closed__1 = _init_l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__1___closed__1); -l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__1___closed__2 = _init_l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__1___closed__2); -l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__2___closed__1 = _init_l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__2___closed__1(); -lean_mark_persistent(l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__2___closed__1); -l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__2___closed__2 = _init_l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__2___closed__2(); -lean_mark_persistent(l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__2___closed__2); -l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__3___closed__1 = _init_l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__3___closed__1(); -lean_mark_persistent(l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__3___closed__1); -l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__3___closed__2 = _init_l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__3___closed__2(); -lean_mark_persistent(l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__3___closed__2); -l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___closed__1 = _init_l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___closed__1(); -lean_mark_persistent(l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___closed__1); -l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___closed__2 = _init_l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___closed__2(); -lean_mark_persistent(l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___closed__2); -l_Lean_Elab_applyVisibility___at_Lean_Elab_Command_expandDeclId___spec__6___closed__1 = _init_l_Lean_Elab_applyVisibility___at_Lean_Elab_Command_expandDeclId___spec__6___closed__1(); -lean_mark_persistent(l_Lean_Elab_applyVisibility___at_Lean_Elab_Command_expandDeclId___spec__6___closed__1); -l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___lambda__2___closed__1 = _init_l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___lambda__2___closed__1(); -lean_mark_persistent(l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___lambda__2___closed__1); -l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___lambda__2___closed__2 = _init_l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___lambda__2___closed__2(); -lean_mark_persistent(l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___lambda__2___closed__2); -l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___closed__1 = _init_l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___closed__1(); -lean_mark_persistent(l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___closed__1); -l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___closed__2 = _init_l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___closed__2(); -lean_mark_persistent(l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___closed__2); -l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___closed__3 = _init_l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___closed__3(); -lean_mark_persistent(l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___closed__3); -l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___closed__4 = _init_l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___closed__4(); -lean_mark_persistent(l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___closed__4); -l_Lean_addDocString___at_Lean_Elab_Command_expandDeclId___spec__14___lambda__1___closed__1 = _init_l_Lean_addDocString___at_Lean_Elab_Command_expandDeclId___spec__14___lambda__1___closed__1(); -lean_mark_persistent(l_Lean_addDocString___at_Lean_Elab_Command_expandDeclId___spec__14___lambda__1___closed__1); -l_Lean_addDocString___at_Lean_Elab_Command_expandDeclId___spec__14___closed__1 = _init_l_Lean_addDocString___at_Lean_Elab_Command_expandDeclId___spec__14___closed__1(); -lean_mark_persistent(l_Lean_addDocString___at_Lean_Elab_Command_expandDeclId___spec__14___closed__1); -l_Lean_addDocString___at_Lean_Elab_Command_expandDeclId___spec__14___closed__2 = _init_l_Lean_addDocString___at_Lean_Elab_Command_expandDeclId___spec__14___closed__2(); -lean_mark_persistent(l_Lean_addDocString___at_Lean_Elab_Command_expandDeclId___spec__14___closed__2); -l_Lean_Elab_expandDeclId___at_Lean_Elab_Command_expandDeclId___spec__1___closed__1 = _init_l_Lean_Elab_expandDeclId___at_Lean_Elab_Command_expandDeclId___spec__1___closed__1(); -lean_mark_persistent(l_Lean_Elab_expandDeclId___at_Lean_Elab_Command_expandDeclId___spec__1___closed__1); -l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__19___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__19___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__19___closed__1); -l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__19___closed__2 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__19___closed__2(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__19___closed__2); -l_Lean_liftCommandElabM___rarg___closed__1 = _init_l_Lean_liftCommandElabM___rarg___closed__1(); -lean_mark_persistent(l_Lean_liftCommandElabM___rarg___closed__1); -l_Lean_liftCommandElabM___rarg___closed__2 = _init_l_Lean_liftCommandElabM___rarg___closed__2(); -lean_mark_persistent(l_Lean_liftCommandElabM___rarg___closed__2); -l_Lean_liftCommandElabM___rarg___closed__3 = _init_l_Lean_liftCommandElabM___rarg___closed__3(); -lean_mark_persistent(l_Lean_liftCommandElabM___rarg___closed__3); -l_Lean_liftCommandElabM___rarg___closed__4 = _init_l_Lean_liftCommandElabM___rarg___closed__4(); -lean_mark_persistent(l_Lean_liftCommandElabM___rarg___closed__4); -l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__4___closed__1 = _init_l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__4___closed__1(); -lean_mark_persistent(l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__4___closed__1); -l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__4___closed__2 = _init_l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__4___closed__2(); -lean_mark_persistent(l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__4___closed__2); +l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___closed__1 = _init_l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___closed__1(); +lean_mark_persistent(l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___closed__1); +l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___closed__2 = _init_l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___closed__2(); +lean_mark_persistent(l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___closed__2); +l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___closed__3 = _init_l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___closed__3(); +lean_mark_persistent(l___private_Lean_Elab_Command_0__Lean_liftCommandElabMCore___rarg___closed__3); +l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6___closed__1 = _init_l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6___closed__1(); +lean_mark_persistent(l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6___closed__1); +l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6___closed__2 = _init_l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6___closed__2(); +lean_mark_persistent(l_Lean_Elab_elabSetOption_setOption___at_Lean_withSetOptionIn___spec__6___closed__2); l_Lean_Elab_elabSetOption___at_Lean_withSetOptionIn___spec__1___closed__1 = _init_l_Lean_Elab_elabSetOption___at_Lean_withSetOptionIn___spec__1___closed__1(); lean_mark_persistent(l_Lean_Elab_elabSetOption___at_Lean_withSetOptionIn___spec__1___closed__1); l_Lean_Elab_elabSetOption___at_Lean_withSetOptionIn___spec__1___closed__2 = _init_l_Lean_Elab_elabSetOption___at_Lean_withSetOptionIn___spec__1___closed__2(); diff --git a/stage0/stdlib/Lean/Elab/ComputedFields.c b/stage0/stdlib/Lean/Elab/ComputedFields.c index bddfa98091f0..15bf8086e5e1 100644 --- a/stage0/stdlib/Lean/Elab/ComputedFields.c +++ b/stage0/stdlib/Lean/Elab/ComputedFields.c @@ -126,7 +126,6 @@ lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withLetDeclImp___rarg(lean static lean_object* l_Lean_Elab_ComputedFields_initFn____x40_Lean_Elab_ComputedFields___hyg_5____closed__2; lean_object* l_Lean_getConstInfo___at___private_Lean_Compiler_InlineAttrs_0__Lean_Compiler_isValidMacroInline___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_ComputedFields_overrideComputedFields___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__3___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_whnfEasyCases___at_Lean_Elab_ComputedFields_getComputedFieldValue___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_ComputedFields_overrideComputedFields___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -202,7 +201,7 @@ uint8_t l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler LEAN_EXPORT lean_object* l_Lean_logAt___at_Lean_Elab_ComputedFields_setComputedFields___spec__2___lambda__2___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescope___at_Lean_Elab_ComputedFields_mkImplType___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_instantiateLevelParams(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Elab_ComputedFields_overrideCasesOn___spec__6___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_compileDecls(lean_object*, lean_object*, lean_object*, lean_object*); @@ -215,7 +214,6 @@ LEAN_EXPORT lean_object* l_Lean_log___at_Lean_Elab_ComputedFields_setComputedFie static lean_object* l_Lean_Elab_ComputedFields_initFn____x40_Lean_Elab_ComputedFields___hyg_5____closed__9; lean_object* l_Array_append___rarg(lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofExpr(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__5___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_getConfig(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallTelescopeReducingAuxAux___rarg(uint8_t, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_LocalDecl_isImplementationDetail(lean_object*); @@ -268,7 +266,6 @@ LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_ComputedFields_setComp lean_object* lean_nat_sub(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_setEnv___at_Lean_Elab_ComputedFields_overrideCasesOn___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_getAppFn(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__5(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_ComputedFields_getComputedFieldValue___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_ComputedFields_overrideCasesOn___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_ComputedFields_initFn____x40_Lean_Elab_ComputedFields___hyg_5____lambda__1___closed__3; @@ -290,7 +287,6 @@ uint8_t l_Lean_Expr_occurs(lean_object*, lean_object*); static lean_object* l_Lean_setImplementedBy___at_Lean_Elab_ComputedFields_overrideCasesOn___spec__8___closed__1; static lean_object* l_Lean_logAt___at_Lean_Elab_ComputedFields_setComputedFields___spec__2___closed__1; size_t lean_usize_add(size_t, size_t); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__3(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_ComputedFields_overrideCasesOn___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescope___at_Lean_Elab_ComputedFields_mkImplType___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_uget(lean_object*, size_t); @@ -304,7 +300,6 @@ lean_object* l_Lean_Meta_setInlineAttribute(lean_object*, uint8_t, lean_object*, lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getConstInfoInduct___at_Lean_Elab_ComputedFields_getComputedFieldValue___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Compiler_implementedByAttr; -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_setImplementedBy___at_Lean_Elab_ComputedFields_overrideConstructors___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_setEnv___at_Lean_Elab_ComputedFields_overrideCasesOn___spec__10___closed__4; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_ComputedFields_validateComputedFields___spec__3(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -316,19 +311,16 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_ComputedFields_ lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_ComputedFields_overrideConstructors___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__5___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkLambdaFVars(lean_object*, lean_object*, uint8_t, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_ComputedFields_overrideComputedFields___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_ComputedFields_setComputedFields___spec__3___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_ComputedFields_mkComputedFieldOverrides___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_ComputedFields_overrideCasesOn(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__4(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_ComputedFields_overrideComputedFields(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_throwError___at_Lean_Attribute_Builtin_ensureNoArgs___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_uset(lean_object*, size_t, lean_object*); lean_object* l_Lean_MessageData_ofName(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__2(lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_instantiateForallAux(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l___private_Lean_Message_0__Lean_beqMessageSeverity____x40_Lean_Message___hyg_106_(uint8_t, uint8_t); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_ComputedFields_overrideComputedFields___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -9507,208 +9499,6 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__3(size_t x_1, size_t x_2, lean_object* x_3) { -_start: -{ -uint8_t x_4; -x_4 = lean_usize_dec_lt(x_2, x_1); -if (x_4 == 0) -{ -return x_3; -} -else -{ -lean_object* x_5; lean_object* x_6; lean_object* x_7; size_t x_8; size_t x_9; uint8_t x_10; -x_5 = lean_array_uget(x_3, x_2); -x_6 = lean_unsigned_to_nat(0u); -x_7 = lean_array_uset(x_3, x_2, x_6); -x_8 = 1; -x_9 = lean_usize_add(x_2, x_8); -x_10 = !lean_is_exclusive(x_5); -if (x_10 == 0) -{ -lean_object* x_11; uint8_t x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_11 = lean_ctor_get(x_5, 0); -x_12 = 0; -x_13 = lean_box(x_12); -lean_ctor_set(x_5, 0, x_13); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_11); -lean_ctor_set(x_14, 1, x_5); -x_15 = lean_array_uset(x_7, x_2, x_14); -x_2 = x_9; -x_3 = x_15; -goto _start; -} -else -{ -lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_17 = lean_ctor_get(x_5, 0); -x_18 = lean_ctor_get(x_5, 1); -lean_inc(x_18); -lean_inc(x_17); -lean_dec(x_5); -x_19 = 0; -x_20 = lean_box(x_19); -x_21 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_21, 0, x_20); -lean_ctor_set(x_21, 1, x_18); -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_17); -lean_ctor_set(x_22, 1, x_21); -x_23 = lean_array_uset(x_7, x_2, x_22); -x_2 = x_9; -x_3 = x_23; -goto _start; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__5___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; lean_object* x_12; -x_11 = lean_array_push(x_1, x_5); -x_12 = l_Lean_Meta_withLocalDecls_loop___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__5___rarg(x_2, x_3, x_4, x_11, x_6, x_7, x_8, x_9, x_10); -return x_12; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__5___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_10 = lean_array_get_size(x_4); -x_11 = lean_array_get_size(x_1); -x_12 = lean_nat_dec_lt(x_10, x_11); -lean_dec(x_11); -if (x_12 == 0) -{ -lean_object* x_13; -lean_dec(x_10); -lean_dec(x_3); -lean_dec(x_1); -x_13 = lean_apply_6(x_2, x_4, x_5, x_6, x_7, x_8, x_9); -return x_13; -} -else -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_14 = lean_array_fget(x_1, x_10); -lean_dec(x_10); -x_15 = lean_ctor_get(x_14, 1); -lean_inc(x_15); -x_16 = lean_ctor_get(x_14, 0); -lean_inc(x_16); -lean_dec(x_14); -x_17 = lean_ctor_get(x_15, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_15, 1); -lean_inc(x_18); -lean_dec(x_15); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -x_19 = lean_apply_6(x_18, x_4, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_19) == 0) -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; uint8_t x_24; lean_object* x_25; -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_19, 1); -lean_inc(x_21); -lean_dec(x_19); -x_22 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecls_loop___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__5___rarg___lambda__1), 10, 4); -lean_closure_set(x_22, 0, x_4); -lean_closure_set(x_22, 1, x_1); -lean_closure_set(x_22, 2, x_2); -lean_closure_set(x_22, 3, x_3); -x_23 = 0; -x_24 = lean_unbox(x_17); -lean_dec(x_17); -x_25 = l_Lean_Meta_withLocalDecl___at_Lean_Meta_GeneralizeTelescope_generalizeTelescopeAux___spec__1___rarg(x_16, x_24, x_20, x_22, x_23, x_5, x_6, x_7, x_8, x_21); -return x_25; -} -else -{ -uint8_t x_26; -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_26 = !lean_is_exclusive(x_19); -if (x_26 == 0) -{ -return x_19; -} -else -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_19, 0); -x_28 = lean_ctor_get(x_19, 1); -lean_inc(x_28); -lean_inc(x_27); -lean_dec(x_19); -x_29 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_29, 0, x_27); -lean_ctor_set(x_29, 1, x_28); -return x_29; -} -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__5(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecls_loop___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__5___rarg), 9, 0); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__4___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; lean_object* x_10; -x_9 = l_List_mapM_loop___at_Lean_Elab_ComputedFields_mkImplType___spec__2___lambda__1___closed__3; -x_10 = l_Lean_Meta_withLocalDecls_loop___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__5___rarg(x_2, x_3, x_1, x_9, x_4, x_5, x_6, x_7, x_8); -return x_10; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__4(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecls___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__4___rarg), 8, 0); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -size_t x_9; size_t x_10; lean_object* x_11; lean_object* x_12; -x_9 = lean_array_size(x_2); -x_10 = 0; -x_11 = l_Array_mapMUnsafe_map___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__3(x_9, x_10, x_2); -x_12 = l_Lean_Meta_withLocalDecls___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__4___rarg(x_1, x_11, x_3, x_4, x_5, x_6, x_7, x_8); -return x_12; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__2(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDeclsD___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__2___rarg), 8, 0); -return x_2; -} -} LEAN_EXPORT lean_object* l_Lean_Elab_ComputedFields_mkComputedFieldOverrides___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { @@ -9915,7 +9705,7 @@ lean_closure_set(x_21, 3, x_3); lean_closure_set(x_21, 4, x_17); lean_closure_set(x_21, 5, x_5); x_22 = l_instInhabitedPUnit; -x_23 = l_Lean_Meta_withLocalDeclsD___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__2___rarg(x_22, x_20, x_21, x_6, x_7, x_8, x_9, x_10); +x_23 = l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__2___rarg(x_22, x_20, x_21, x_6, x_7, x_8, x_9, x_10); return x_23; } } @@ -10090,18 +9880,6 @@ x_9 = l_Array_mapMUnsafe_map___at_Lean_Elab_ComputedFields_mkComputedFieldOverri return x_9; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -size_t x_4; size_t x_5; lean_object* x_6; -x_4 = lean_unbox_usize(x_1); -lean_dec(x_1); -x_5 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_6 = l_Array_mapMUnsafe_map___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__3(x_4, x_5, x_3); -return x_6; -} -} LEAN_EXPORT lean_object* l_Lean_Elab_ComputedFields_mkComputedFieldOverrides___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { diff --git a/stage0/stdlib/Lean/Elab/DeclModifiers.c b/stage0/stdlib/Lean/Elab/DeclModifiers.c index 89c360f5591b..c4de9ab6a254 100644 --- a/stage0/stdlib/Lean/Elab/DeclModifiers.c +++ b/stage0/stdlib/Lean/Elab/DeclModifiers.c @@ -33,7 +33,7 @@ static lean_object* l_Lean_Elab_expandOptDocComment_x3f___rarg___closed__1; lean_object* lean_private_to_user_name(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_checkIfShadowingStructureField___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Elab_checkNotAlreadyDeclared___rarg___lambda__1___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*); static lean_object* l_Lean_Elab_Modifiers_filterAttrs___closed__1; static lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__3___closed__7; static lean_object* l_Lean_Elab_instToStringVisibility___closed__2; @@ -42,7 +42,7 @@ lean_object* l_Lean_Syntax_formatStxAux(lean_object*, uint8_t, lean_object*, lea LEAN_EXPORT lean_object* l_Lean_Elab_expandDeclId___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_expandDeclIdCore___closed__3; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_checkIfShadowingStructureField___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); static lean_object* l_Lean_Elab_instToFormatModifiers___closed__3; static lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__3___closed__6; lean_object* l_Lean_Name_toString(lean_object*, uint8_t, lean_object*); @@ -58,7 +58,6 @@ static lean_object* l_Lean_Elab_applyVisibility___rarg___lambda__2___closed__1; uint8_t lean_usize_dec_eq(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Elab_instToStringModifiers___lambda__1(lean_object*); lean_object* l_Lean_Syntax_getArgs(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_instToFormatModifiers___closed__9; static lean_object* l_Lean_Elab_mkDeclName___rarg___closed__3; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_expandDeclId___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); @@ -97,7 +96,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_checkIfShadowingStructureField___rarg___lam static lean_object* l_Lean_Elab_checkNotAlreadyDeclared___rarg___lambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_RecKind_noConfusion(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Visibility_toCtorIdx___boxed(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__3(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_isReservedName(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__2___boxed(lean_object**); LEAN_EXPORT lean_object* l_Lean_Elab_RecKind_toCtorIdx___boxed(lean_object*); @@ -274,7 +273,7 @@ uint8_t lean_nat_dec_le(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Modifiers_filterAttrs___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); static lean_object* l_Lean_Elab_instToFormatModifiers___closed__29; -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_checkIfShadowingStructureField___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_instToFormatModifiers___closed__24; static lean_object* l_Lean_Elab_checkNotAlreadyDeclared___rarg___lambda__1___closed__1; @@ -1175,20 +1174,22 @@ return x_2; static lean_object* _init_l_Lean_Elab_instInhabitedModifiers___closed__2() { _start: { -lean_object* x_1; uint8_t x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; +lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; uint8_t x_5; lean_object* x_6; lean_object* x_7; x_1 = lean_box(0); -x_2 = 0; +x_2 = lean_box(0); x_3 = 0; x_4 = 0; -x_5 = l_Lean_Elab_instInhabitedModifiers___closed__1; -x_6 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_6, 0, x_1); -lean_ctor_set(x_6, 1, x_5); -lean_ctor_set_uint8(x_6, sizeof(void*)*2, x_2); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 1, x_3); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 2, x_4); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 3, x_3); -return x_6; +x_5 = 0; +x_6 = l_Lean_Elab_instInhabitedModifiers___closed__1; +x_7 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_7, 0, x_2); +lean_ctor_set(x_7, 1, x_1); +lean_ctor_set(x_7, 2, x_6); +lean_ctor_set_uint8(x_7, sizeof(void*)*3, x_3); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 1, x_4); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 2, x_5); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 3, x_4); +return x_7; } } static lean_object* _init_l_Lean_Elab_instInhabitedModifiers() { @@ -1203,7 +1204,7 @@ LEAN_EXPORT uint8_t l_Lean_Elab_Modifiers_isPrivate(lean_object* x_1) { _start: { uint8_t x_2; lean_object* x_3; -x_2 = lean_ctor_get_uint8(x_1, sizeof(void*)*2); +x_2 = lean_ctor_get_uint8(x_1, sizeof(void*)*3); x_3 = lean_box(x_2); if (lean_obj_tag(x_3) == 2) { @@ -1234,7 +1235,7 @@ LEAN_EXPORT uint8_t l_Lean_Elab_Modifiers_isProtected(lean_object* x_1) { _start: { uint8_t x_2; lean_object* x_3; -x_2 = lean_ctor_get_uint8(x_1, sizeof(void*)*2); +x_2 = lean_ctor_get_uint8(x_1, sizeof(void*)*3); x_3 = lean_box(x_2); if (lean_obj_tag(x_3) == 1) { @@ -1265,7 +1266,7 @@ LEAN_EXPORT uint8_t l_Lean_Elab_Modifiers_isPartial(lean_object* x_1) { _start: { uint8_t x_2; lean_object* x_3; -x_2 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 2); +x_2 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 2); x_3 = lean_box(x_2); if (lean_obj_tag(x_3) == 0) { @@ -1296,7 +1297,7 @@ LEAN_EXPORT uint8_t l_Lean_Elab_Modifiers_isNonrec(lean_object* x_1) { _start: { uint8_t x_2; lean_object* x_3; -x_2 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 2); +x_2 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 2); x_3 = lean_box(x_2); if (lean_obj_tag(x_3) == 1) { @@ -1331,32 +1332,35 @@ x_3 = !lean_is_exclusive(x_1); if (x_3 == 0) { lean_object* x_4; lean_object* x_5; -x_4 = lean_ctor_get(x_1, 1); +x_4 = lean_ctor_get(x_1, 2); x_5 = lean_array_push(x_4, x_2); -lean_ctor_set(x_1, 1, x_5); +lean_ctor_set(x_1, 2, x_5); return x_1; } else { -lean_object* x_6; uint8_t x_7; uint8_t x_8; uint8_t x_9; uint8_t x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +lean_object* x_6; lean_object* x_7; uint8_t x_8; uint8_t x_9; uint8_t x_10; uint8_t x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; x_6 = lean_ctor_get(x_1, 0); -x_7 = lean_ctor_get_uint8(x_1, sizeof(void*)*2); -x_8 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 1); -x_9 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 2); -x_10 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 3); -x_11 = lean_ctor_get(x_1, 1); -lean_inc(x_11); +x_7 = lean_ctor_get(x_1, 1); +x_8 = lean_ctor_get_uint8(x_1, sizeof(void*)*3); +x_9 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 1); +x_10 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 2); +x_11 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 3); +x_12 = lean_ctor_get(x_1, 2); +lean_inc(x_12); +lean_inc(x_7); lean_inc(x_6); lean_dec(x_1); -x_12 = lean_array_push(x_11, x_2); -x_13 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_13, 0, x_6); -lean_ctor_set(x_13, 1, x_12); -lean_ctor_set_uint8(x_13, sizeof(void*)*2, x_7); -lean_ctor_set_uint8(x_13, sizeof(void*)*2 + 1, x_8); -lean_ctor_set_uint8(x_13, sizeof(void*)*2 + 2, x_9); -lean_ctor_set_uint8(x_13, sizeof(void*)*2 + 3, x_10); -return x_13; +x_13 = lean_array_push(x_12, x_2); +x_14 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_14, 0, x_6); +lean_ctor_set(x_14, 1, x_7); +lean_ctor_set(x_14, 2, x_13); +lean_ctor_set_uint8(x_14, sizeof(void*)*3, x_8); +lean_ctor_set_uint8(x_14, sizeof(void*)*3 + 1, x_9); +lean_ctor_set_uint8(x_14, sizeof(void*)*3 + 2, x_10); +lean_ctor_set_uint8(x_14, sizeof(void*)*3 + 3, x_11); +return x_14; } } } @@ -1415,7 +1419,7 @@ x_3 = !lean_is_exclusive(x_1); if (x_3 == 0) { lean_object* x_4; lean_object* x_5; lean_object* x_6; uint8_t x_7; -x_4 = lean_ctor_get(x_1, 1); +x_4 = lean_ctor_get(x_1, 2); x_5 = lean_array_get_size(x_4); x_6 = lean_unsigned_to_nat(0u); x_7 = lean_nat_dec_lt(x_6, x_5); @@ -1426,7 +1430,7 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); x_8 = l_Lean_Elab_Modifiers_filterAttrs___closed__1; -lean_ctor_set(x_1, 1, x_8); +lean_ctor_set(x_1, 2, x_8); return x_1; } else @@ -1440,7 +1444,7 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); x_10 = l_Lean_Elab_Modifiers_filterAttrs___closed__1; -lean_ctor_set(x_1, 1, x_10); +lean_ctor_set(x_1, 2, x_10); return x_1; } else @@ -1452,79 +1456,84 @@ lean_dec(x_5); x_13 = l_Lean_Elab_Modifiers_filterAttrs___closed__1; x_14 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Modifiers_filterAttrs___spec__1(x_2, x_4, x_11, x_12, x_13); lean_dec(x_4); -lean_ctor_set(x_1, 1, x_14); +lean_ctor_set(x_1, 2, x_14); return x_1; } } } else { -lean_object* x_15; uint8_t x_16; uint8_t x_17; uint8_t x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; +lean_object* x_15; lean_object* x_16; uint8_t x_17; uint8_t x_18; uint8_t x_19; uint8_t x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; x_15 = lean_ctor_get(x_1, 0); -x_16 = lean_ctor_get_uint8(x_1, sizeof(void*)*2); -x_17 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 1); -x_18 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 2); -x_19 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 3); -x_20 = lean_ctor_get(x_1, 1); -lean_inc(x_20); +x_16 = lean_ctor_get(x_1, 1); +x_17 = lean_ctor_get_uint8(x_1, sizeof(void*)*3); +x_18 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 1); +x_19 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 2); +x_20 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 3); +x_21 = lean_ctor_get(x_1, 2); +lean_inc(x_21); +lean_inc(x_16); lean_inc(x_15); lean_dec(x_1); -x_21 = lean_array_get_size(x_20); -x_22 = lean_unsigned_to_nat(0u); -x_23 = lean_nat_dec_lt(x_22, x_21); -if (x_23 == 0) +x_22 = lean_array_get_size(x_21); +x_23 = lean_unsigned_to_nat(0u); +x_24 = lean_nat_dec_lt(x_23, x_22); +if (x_24 == 0) { -lean_object* x_24; lean_object* x_25; +lean_object* x_25; lean_object* x_26; +lean_dec(x_22); lean_dec(x_21); -lean_dec(x_20); lean_dec(x_2); -x_24 = l_Lean_Elab_Modifiers_filterAttrs___closed__1; -x_25 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_25, 0, x_15); -lean_ctor_set(x_25, 1, x_24); -lean_ctor_set_uint8(x_25, sizeof(void*)*2, x_16); -lean_ctor_set_uint8(x_25, sizeof(void*)*2 + 1, x_17); -lean_ctor_set_uint8(x_25, sizeof(void*)*2 + 2, x_18); -lean_ctor_set_uint8(x_25, sizeof(void*)*2 + 3, x_19); -return x_25; +x_25 = l_Lean_Elab_Modifiers_filterAttrs___closed__1; +x_26 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_26, 0, x_15); +lean_ctor_set(x_26, 1, x_16); +lean_ctor_set(x_26, 2, x_25); +lean_ctor_set_uint8(x_26, sizeof(void*)*3, x_17); +lean_ctor_set_uint8(x_26, sizeof(void*)*3 + 1, x_18); +lean_ctor_set_uint8(x_26, sizeof(void*)*3 + 2, x_19); +lean_ctor_set_uint8(x_26, sizeof(void*)*3 + 3, x_20); +return x_26; } else { -uint8_t x_26; -x_26 = lean_nat_dec_le(x_21, x_21); -if (x_26 == 0) +uint8_t x_27; +x_27 = lean_nat_dec_le(x_22, x_22); +if (x_27 == 0) { -lean_object* x_27; lean_object* x_28; +lean_object* x_28; lean_object* x_29; +lean_dec(x_22); lean_dec(x_21); -lean_dec(x_20); lean_dec(x_2); -x_27 = l_Lean_Elab_Modifiers_filterAttrs___closed__1; -x_28 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_28, 0, x_15); -lean_ctor_set(x_28, 1, x_27); -lean_ctor_set_uint8(x_28, sizeof(void*)*2, x_16); -lean_ctor_set_uint8(x_28, sizeof(void*)*2 + 1, x_17); -lean_ctor_set_uint8(x_28, sizeof(void*)*2 + 2, x_18); -lean_ctor_set_uint8(x_28, sizeof(void*)*2 + 3, x_19); -return x_28; +x_28 = l_Lean_Elab_Modifiers_filterAttrs___closed__1; +x_29 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_29, 0, x_15); +lean_ctor_set(x_29, 1, x_16); +lean_ctor_set(x_29, 2, x_28); +lean_ctor_set_uint8(x_29, sizeof(void*)*3, x_17); +lean_ctor_set_uint8(x_29, sizeof(void*)*3 + 1, x_18); +lean_ctor_set_uint8(x_29, sizeof(void*)*3 + 2, x_19); +lean_ctor_set_uint8(x_29, sizeof(void*)*3 + 3, x_20); +return x_29; } else { -size_t x_29; size_t x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_29 = 0; -x_30 = lean_usize_of_nat(x_21); +size_t x_30; size_t x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_30 = 0; +x_31 = lean_usize_of_nat(x_22); +lean_dec(x_22); +x_32 = l_Lean_Elab_Modifiers_filterAttrs___closed__1; +x_33 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Modifiers_filterAttrs___spec__1(x_2, x_21, x_30, x_31, x_32); lean_dec(x_21); -x_31 = l_Lean_Elab_Modifiers_filterAttrs___closed__1; -x_32 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Modifiers_filterAttrs___spec__1(x_2, x_20, x_29, x_30, x_31); -lean_dec(x_20); -x_33 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_33, 0, x_15); -lean_ctor_set(x_33, 1, x_32); -lean_ctor_set_uint8(x_33, sizeof(void*)*2, x_16); -lean_ctor_set_uint8(x_33, sizeof(void*)*2 + 1, x_17); -lean_ctor_set_uint8(x_33, sizeof(void*)*2 + 2, x_18); -lean_ctor_set_uint8(x_33, sizeof(void*)*2 + 3, x_19); -return x_33; +x_34 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_34, 0, x_15); +lean_ctor_set(x_34, 1, x_16); +lean_ctor_set(x_34, 2, x_33); +lean_ctor_set_uint8(x_34, sizeof(void*)*3, x_17); +lean_ctor_set_uint8(x_34, sizeof(void*)*3 + 1, x_18); +lean_ctor_set_uint8(x_34, sizeof(void*)*3 + 2, x_19); +lean_ctor_set_uint8(x_34, sizeof(void*)*3 + 3, x_20); +return x_34; } } } @@ -2055,13 +2064,13 @@ LEAN_EXPORT lean_object* l_Lean_Elab_instToFormatModifiers(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; uint8_t x_4; uint8_t x_5; uint8_t x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_2 = lean_ctor_get(x_1, 0); +x_2 = lean_ctor_get(x_1, 1); lean_inc(x_2); -x_3 = lean_ctor_get_uint8(x_1, sizeof(void*)*2); -x_4 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 1); -x_5 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 2); -x_6 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 3); -x_7 = lean_ctor_get(x_1, 1); +x_3 = lean_ctor_get_uint8(x_1, sizeof(void*)*3); +x_4 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 1); +x_5 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 2); +x_6 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 3); +x_7 = lean_ctor_get(x_1, 2); lean_inc(x_7); lean_dec(x_1); x_8 = lean_array_to_list(x_7); @@ -2267,13 +2276,13 @@ LEAN_EXPORT lean_object* l_Lean_Elab_instToStringModifiers___lambda__2(lean_obje _start: { lean_object* x_2; uint8_t x_3; uint8_t x_4; uint8_t x_5; uint8_t x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_2 = lean_ctor_get(x_1, 0); +x_2 = lean_ctor_get(x_1, 1); lean_inc(x_2); -x_3 = lean_ctor_get_uint8(x_1, sizeof(void*)*2); -x_4 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 1); -x_5 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 2); -x_6 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 3); -x_7 = lean_ctor_get(x_1, 1); +x_3 = lean_ctor_get_uint8(x_1, sizeof(void*)*3); +x_4 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 1); +x_5 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 2); +x_6 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 3); +x_7 = lean_ctor_get(x_1, 2); lean_inc(x_7); lean_dec(x_1); x_8 = lean_array_to_list(x_7); @@ -2662,102 +2671,108 @@ lean_dec(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, uint8_t x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, uint8_t x_6, uint8_t x_7, lean_object* x_8) { _start: { -lean_object* x_8; lean_object* x_9; uint8_t x_10; uint8_t x_11; -x_8 = lean_ctor_get(x_1, 0); -lean_inc(x_8); -lean_dec(x_1); -x_9 = lean_ctor_get(x_8, 1); +lean_object* x_9; lean_object* x_10; uint8_t x_11; uint8_t x_12; +x_9 = lean_ctor_get(x_1, 0); lean_inc(x_9); -lean_dec(x_8); -x_10 = l_Lean_Syntax_isNone(x_2); -x_11 = l_Lean_Syntax_isNone(x_3); -if (x_10 == 0) -{ +lean_dec(x_1); +x_10 = lean_ctor_get(x_9, 1); +lean_inc(x_10); +lean_dec(x_9); +x_11 = l_Lean_Syntax_isNone(x_2); +x_12 = l_Lean_Syntax_isNone(x_3); if (x_11 == 0) { -uint8_t x_12; lean_object* x_13; lean_object* x_14; -x_12 = 1; -x_13 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_13, 0, x_4); -lean_ctor_set(x_13, 1, x_7); -lean_ctor_set_uint8(x_13, sizeof(void*)*2, x_5); -lean_ctor_set_uint8(x_13, sizeof(void*)*2 + 1, x_12); -lean_ctor_set_uint8(x_13, sizeof(void*)*2 + 2, x_6); -lean_ctor_set_uint8(x_13, sizeof(void*)*2 + 3, x_12); -x_14 = lean_apply_2(x_9, lean_box(0), x_13); -return x_14; +if (x_12 == 0) +{ +uint8_t x_13; lean_object* x_14; lean_object* x_15; +x_13 = 1; +x_14 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_14, 0, x_4); +lean_ctor_set(x_14, 1, x_5); +lean_ctor_set(x_14, 2, x_8); +lean_ctor_set_uint8(x_14, sizeof(void*)*3, x_6); +lean_ctor_set_uint8(x_14, sizeof(void*)*3 + 1, x_13); +lean_ctor_set_uint8(x_14, sizeof(void*)*3 + 2, x_7); +lean_ctor_set_uint8(x_14, sizeof(void*)*3 + 3, x_13); +x_15 = lean_apply_2(x_10, lean_box(0), x_14); +return x_15; } else { -uint8_t x_15; uint8_t x_16; lean_object* x_17; lean_object* x_18; -x_15 = 1; -x_16 = 0; -x_17 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_17, 0, x_4); -lean_ctor_set(x_17, 1, x_7); -lean_ctor_set_uint8(x_17, sizeof(void*)*2, x_5); -lean_ctor_set_uint8(x_17, sizeof(void*)*2 + 1, x_15); -lean_ctor_set_uint8(x_17, sizeof(void*)*2 + 2, x_6); -lean_ctor_set_uint8(x_17, sizeof(void*)*2 + 3, x_16); -x_18 = lean_apply_2(x_9, lean_box(0), x_17); -return x_18; +uint8_t x_16; uint8_t x_17; lean_object* x_18; lean_object* x_19; +x_16 = 1; +x_17 = 0; +x_18 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_18, 0, x_4); +lean_ctor_set(x_18, 1, x_5); +lean_ctor_set(x_18, 2, x_8); +lean_ctor_set_uint8(x_18, sizeof(void*)*3, x_6); +lean_ctor_set_uint8(x_18, sizeof(void*)*3 + 1, x_16); +lean_ctor_set_uint8(x_18, sizeof(void*)*3 + 2, x_7); +lean_ctor_set_uint8(x_18, sizeof(void*)*3 + 3, x_17); +x_19 = lean_apply_2(x_10, lean_box(0), x_18); +return x_19; } } else { -if (x_11 == 0) +if (x_12 == 0) { -uint8_t x_19; uint8_t x_20; lean_object* x_21; lean_object* x_22; -x_19 = 0; -x_20 = 1; -x_21 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_21, 0, x_4); -lean_ctor_set(x_21, 1, x_7); -lean_ctor_set_uint8(x_21, sizeof(void*)*2, x_5); -lean_ctor_set_uint8(x_21, sizeof(void*)*2 + 1, x_19); -lean_ctor_set_uint8(x_21, sizeof(void*)*2 + 2, x_6); -lean_ctor_set_uint8(x_21, sizeof(void*)*2 + 3, x_20); -x_22 = lean_apply_2(x_9, lean_box(0), x_21); -return x_22; +uint8_t x_20; uint8_t x_21; lean_object* x_22; lean_object* x_23; +x_20 = 0; +x_21 = 1; +x_22 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_22, 0, x_4); +lean_ctor_set(x_22, 1, x_5); +lean_ctor_set(x_22, 2, x_8); +lean_ctor_set_uint8(x_22, sizeof(void*)*3, x_6); +lean_ctor_set_uint8(x_22, sizeof(void*)*3 + 1, x_20); +lean_ctor_set_uint8(x_22, sizeof(void*)*3 + 2, x_7); +lean_ctor_set_uint8(x_22, sizeof(void*)*3 + 3, x_21); +x_23 = lean_apply_2(x_10, lean_box(0), x_22); +return x_23; } else { -uint8_t x_23; lean_object* x_24; lean_object* x_25; -x_23 = 0; -x_24 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_24, 0, x_4); -lean_ctor_set(x_24, 1, x_7); -lean_ctor_set_uint8(x_24, sizeof(void*)*2, x_5); -lean_ctor_set_uint8(x_24, sizeof(void*)*2 + 1, x_23); -lean_ctor_set_uint8(x_24, sizeof(void*)*2 + 2, x_6); -lean_ctor_set_uint8(x_24, sizeof(void*)*2 + 3, x_23); -x_25 = lean_apply_2(x_9, lean_box(0), x_24); -return x_25; +uint8_t x_24; lean_object* x_25; lean_object* x_26; +x_24 = 0; +x_25 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_25, 0, x_4); +lean_ctor_set(x_25, 1, x_5); +lean_ctor_set(x_25, 2, x_8); +lean_ctor_set_uint8(x_25, sizeof(void*)*3, x_6); +lean_ctor_set_uint8(x_25, sizeof(void*)*3 + 1, x_24); +lean_ctor_set_uint8(x_25, sizeof(void*)*3 + 2, x_7); +lean_ctor_set_uint8(x_25, sizeof(void*)*3 + 3, x_24); +x_26 = lean_apply_2(x_10, lean_box(0), x_25); +return x_26; } } } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, uint8_t x_17) { +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, uint8_t x_18) { _start: { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_18 = lean_box(x_17); -x_19 = lean_box(x_5); +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_19 = lean_box(x_18); +x_20 = lean_box(x_6); lean_inc(x_1); -x_20 = lean_alloc_closure((void*)(l_Lean_Elab_elabModifiers___rarg___lambda__1___boxed), 7, 6); -lean_closure_set(x_20, 0, x_1); -lean_closure_set(x_20, 1, x_2); -lean_closure_set(x_20, 2, x_3); -lean_closure_set(x_20, 3, x_4); -lean_closure_set(x_20, 4, x_18); -lean_closure_set(x_20, 5, x_19); -x_21 = l_Lean_Syntax_getOptional_x3f(x_6); -if (lean_obj_tag(x_21) == 0) -{ -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_21 = lean_alloc_closure((void*)(l_Lean_Elab_elabModifiers___rarg___lambda__1___boxed), 8, 7); +lean_closure_set(x_21, 0, x_1); +lean_closure_set(x_21, 1, x_2); +lean_closure_set(x_21, 2, x_3); +lean_closure_set(x_21, 3, x_4); +lean_closure_set(x_21, 4, x_5); +lean_closure_set(x_21, 5, x_19); +lean_closure_set(x_21, 6, x_20); +x_22 = l_Lean_Syntax_getOptional_x3f(x_7); +if (lean_obj_tag(x_22) == 0) +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +lean_dec(x_17); lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); @@ -2767,32 +2782,31 @@ lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_7); -x_22 = lean_ctor_get(x_1, 1); -lean_inc(x_22); -x_23 = lean_ctor_get(x_1, 0); +x_23 = lean_ctor_get(x_1, 1); lean_inc(x_23); -lean_dec(x_1); -x_24 = lean_ctor_get(x_23, 1); +x_24 = lean_ctor_get(x_1, 0); lean_inc(x_24); -lean_dec(x_23); -x_25 = l_Lean_Elab_Modifiers_filterAttrs___closed__1; -x_26 = lean_apply_2(x_24, lean_box(0), x_25); -x_27 = lean_apply_4(x_22, lean_box(0), lean_box(0), x_26, x_20); -return x_27; +lean_dec(x_1); +x_25 = lean_ctor_get(x_24, 1); +lean_inc(x_25); +lean_dec(x_24); +x_26 = l_Lean_Elab_Modifiers_filterAttrs___closed__1; +x_27 = lean_apply_2(x_25, lean_box(0), x_26); +x_28 = lean_apply_4(x_23, lean_box(0), lean_box(0), x_27, x_21); +return x_28; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_28 = lean_ctor_get(x_21, 0); -lean_inc(x_28); -lean_dec(x_21); -x_29 = lean_ctor_get(x_1, 1); +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_29 = lean_ctor_get(x_22, 0); lean_inc(x_29); -x_30 = l_Lean_Elab_elabDeclAttrs___rarg(x_1, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_28); -lean_dec(x_28); -x_31 = lean_apply_4(x_29, lean_box(0), lean_box(0), x_30, x_20); -return x_31; +lean_dec(x_22); +x_30 = lean_ctor_get(x_1, 1); +lean_inc(x_30); +x_31 = l_Lean_Elab_elabDeclAttrs___rarg(x_1, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_29); +lean_dec(x_29); +x_32 = lean_apply_4(x_30, lean_box(0), lean_box(0), x_31, x_21); +return x_32; } } } @@ -2861,114 +2875,115 @@ x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18) { _start: { -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_box(x_4); -lean_inc(x_8); +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_box(x_5); +lean_inc(x_9); lean_inc(x_1); -x_19 = lean_alloc_closure((void*)(l_Lean_Elab_elabModifiers___rarg___lambda__2___boxed), 17, 16); -lean_closure_set(x_19, 0, x_1); -lean_closure_set(x_19, 1, x_2); -lean_closure_set(x_19, 2, x_3); -lean_closure_set(x_19, 3, x_17); -lean_closure_set(x_19, 4, x_18); -lean_closure_set(x_19, 5, x_5); -lean_closure_set(x_19, 6, x_6); -lean_closure_set(x_19, 7, x_7); -lean_closure_set(x_19, 8, x_8); -lean_closure_set(x_19, 9, x_9); -lean_closure_set(x_19, 10, x_10); -lean_closure_set(x_19, 11, x_11); -lean_closure_set(x_19, 12, x_12); -lean_closure_set(x_19, 13, x_13); -lean_closure_set(x_19, 14, x_14); -lean_closure_set(x_19, 15, x_15); -x_20 = l_Lean_Syntax_getOptional_x3f(x_16); -if (lean_obj_tag(x_20) == 0) -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; -lean_dec(x_8); -x_21 = lean_ctor_get(x_1, 1); -lean_inc(x_21); -x_22 = lean_ctor_get(x_1, 0); +x_20 = lean_alloc_closure((void*)(l_Lean_Elab_elabModifiers___rarg___lambda__2___boxed), 18, 17); +lean_closure_set(x_20, 0, x_1); +lean_closure_set(x_20, 1, x_2); +lean_closure_set(x_20, 2, x_3); +lean_closure_set(x_20, 3, x_4); +lean_closure_set(x_20, 4, x_18); +lean_closure_set(x_20, 5, x_19); +lean_closure_set(x_20, 6, x_6); +lean_closure_set(x_20, 7, x_7); +lean_closure_set(x_20, 8, x_8); +lean_closure_set(x_20, 9, x_9); +lean_closure_set(x_20, 10, x_10); +lean_closure_set(x_20, 11, x_11); +lean_closure_set(x_20, 12, x_12); +lean_closure_set(x_20, 13, x_13); +lean_closure_set(x_20, 14, x_14); +lean_closure_set(x_20, 15, x_15); +lean_closure_set(x_20, 16, x_16); +x_21 = l_Lean_Syntax_getOptional_x3f(x_17); +if (lean_obj_tag(x_21) == 0) +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +lean_dec(x_9); +x_22 = lean_ctor_get(x_1, 1); lean_inc(x_22); -lean_dec(x_1); -x_23 = lean_ctor_get(x_22, 1); +x_23 = lean_ctor_get(x_1, 0); lean_inc(x_23); -lean_dec(x_22); -x_24 = 0; -x_25 = lean_box(x_24); -x_26 = lean_apply_2(x_23, lean_box(0), x_25); -x_27 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_26, x_19); -return x_27; +lean_dec(x_1); +x_24 = lean_ctor_get(x_23, 1); +lean_inc(x_24); +lean_dec(x_23); +x_25 = 0; +x_26 = lean_box(x_25); +x_27 = lean_apply_2(x_24, lean_box(0), x_26); +x_28 = lean_apply_4(x_22, lean_box(0), lean_box(0), x_27, x_20); +return x_28; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; -x_28 = lean_ctor_get(x_20, 0); -lean_inc(x_28); -lean_dec(x_20); -lean_inc(x_28); -x_29 = l_Lean_Syntax_getKind(x_28); -x_30 = l_Lean_Elab_elabModifiers___rarg___lambda__3___closed__4; -x_31 = lean_name_eq(x_29, x_30); -if (x_31 == 0) -{ -lean_object* x_32; uint8_t x_33; -x_32 = l_Lean_Elab_elabModifiers___rarg___lambda__3___closed__5; -x_33 = lean_name_eq(x_29, x_32); -lean_dec(x_29); -if (x_33 == 0) -{ -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_34 = lean_ctor_get(x_1, 1); -lean_inc(x_34); -x_35 = l_Lean_Elab_elabModifiers___rarg___lambda__3___closed__7; -x_36 = l_Lean_throwErrorAt___rarg(x_1, x_8, x_28, x_35); -x_37 = lean_apply_4(x_34, lean_box(0), lean_box(0), x_36, x_19); -return x_37; +lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; +x_29 = lean_ctor_get(x_21, 0); +lean_inc(x_29); +lean_dec(x_21); +lean_inc(x_29); +x_30 = l_Lean_Syntax_getKind(x_29); +x_31 = l_Lean_Elab_elabModifiers___rarg___lambda__3___closed__4; +x_32 = lean_name_eq(x_30, x_31); +if (x_32 == 0) +{ +lean_object* x_33; uint8_t x_34; +x_33 = l_Lean_Elab_elabModifiers___rarg___lambda__3___closed__5; +x_34 = lean_name_eq(x_30, x_33); +lean_dec(x_30); +if (x_34 == 0) +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_35 = lean_ctor_get(x_1, 1); +lean_inc(x_35); +x_36 = l_Lean_Elab_elabModifiers___rarg___lambda__3___closed__7; +x_37 = l_Lean_throwErrorAt___rarg(x_1, x_9, x_29, x_36); +x_38 = lean_apply_4(x_35, lean_box(0), lean_box(0), x_37, x_20); +return x_38; } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; -lean_dec(x_28); -lean_dec(x_8); -x_38 = lean_ctor_get(x_1, 1); -lean_inc(x_38); -x_39 = lean_ctor_get(x_1, 0); +lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; +lean_dec(x_29); +lean_dec(x_9); +x_39 = lean_ctor_get(x_1, 1); lean_inc(x_39); -lean_dec(x_1); -x_40 = lean_ctor_get(x_39, 1); +x_40 = lean_ctor_get(x_1, 0); lean_inc(x_40); -lean_dec(x_39); -x_41 = 1; -x_42 = lean_box(x_41); -x_43 = lean_apply_2(x_40, lean_box(0), x_42); -x_44 = lean_apply_4(x_38, lean_box(0), lean_box(0), x_43, x_19); -return x_44; +lean_dec(x_1); +x_41 = lean_ctor_get(x_40, 1); +lean_inc(x_41); +lean_dec(x_40); +x_42 = 1; +x_43 = lean_box(x_42); +x_44 = lean_apply_2(x_41, lean_box(0), x_43); +x_45 = lean_apply_4(x_39, lean_box(0), lean_box(0), x_44, x_20); +return x_45; } } else { -lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; +lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +lean_dec(x_30); lean_dec(x_29); -lean_dec(x_28); -lean_dec(x_8); -x_45 = lean_ctor_get(x_1, 1); -lean_inc(x_45); -x_46 = lean_ctor_get(x_1, 0); +lean_dec(x_9); +x_46 = lean_ctor_get(x_1, 1); lean_inc(x_46); -lean_dec(x_1); -x_47 = lean_ctor_get(x_46, 1); +x_47 = lean_ctor_get(x_1, 0); lean_inc(x_47); -lean_dec(x_46); -x_48 = 2; -x_49 = lean_box(x_48); -x_50 = lean_apply_2(x_47, lean_box(0), x_49); -x_51 = lean_apply_4(x_45, lean_box(0), lean_box(0), x_50, x_19); -return x_51; +lean_dec(x_1); +x_48 = lean_ctor_get(x_47, 1); +lean_inc(x_48); +lean_dec(x_47); +x_49 = 2; +x_50 = lean_box(x_49); +x_51 = lean_apply_2(x_48, lean_box(0), x_50); +x_52 = lean_apply_4(x_46, lean_box(0), lean_box(0), x_51, x_20); +return x_52; } } } @@ -3059,23 +3074,24 @@ lean_object* x_28; lean_object* x_29; x_28 = lean_box(x_27); lean_inc(x_4); lean_inc(x_1); -x_29 = lean_alloc_closure((void*)(l_Lean_Elab_elabModifiers___rarg___lambda__3___boxed), 17, 16); +x_29 = lean_alloc_closure((void*)(l_Lean_Elab_elabModifiers___rarg___lambda__3___boxed), 18, 17); lean_closure_set(x_29, 0, x_1); lean_closure_set(x_29, 1, x_20); lean_closure_set(x_29, 2, x_22); -lean_closure_set(x_29, 3, x_28); -lean_closure_set(x_29, 4, x_16); -lean_closure_set(x_29, 5, x_2); -lean_closure_set(x_29, 6, x_3); -lean_closure_set(x_29, 7, x_4); -lean_closure_set(x_29, 8, x_5); -lean_closure_set(x_29, 9, x_6); -lean_closure_set(x_29, 10, x_7); -lean_closure_set(x_29, 11, x_8); -lean_closure_set(x_29, 12, x_9); -lean_closure_set(x_29, 13, x_10); -lean_closure_set(x_29, 14, x_11); -lean_closure_set(x_29, 15, x_18); +lean_closure_set(x_29, 3, x_12); +lean_closure_set(x_29, 4, x_28); +lean_closure_set(x_29, 5, x_16); +lean_closure_set(x_29, 6, x_2); +lean_closure_set(x_29, 7, x_3); +lean_closure_set(x_29, 8, x_4); +lean_closure_set(x_29, 9, x_5); +lean_closure_set(x_29, 10, x_6); +lean_closure_set(x_29, 11, x_7); +lean_closure_set(x_29, 12, x_8); +lean_closure_set(x_29, 13, x_9); +lean_closure_set(x_29, 14, x_10); +lean_closure_set(x_29, 15, x_11); +lean_closure_set(x_29, 16, x_18); if (lean_obj_tag(x_26) == 0) { lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; @@ -3118,22 +3134,22 @@ LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Elab_elabModifiers___rarg___boxed), 12, 0); +x_2 = lean_alloc_closure((void*)(l_Lean_Elab_elabModifiers___rarg), 12, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -uint8_t x_8; uint8_t x_9; lean_object* x_10; -x_8 = lean_unbox(x_5); -lean_dec(x_5); +uint8_t x_9; uint8_t x_10; lean_object* x_11; x_9 = lean_unbox(x_6); lean_dec(x_6); -x_10 = l_Lean_Elab_elabModifiers___rarg___lambda__1(x_1, x_2, x_3, x_4, x_8, x_9, x_7); +x_10 = lean_unbox(x_7); +lean_dec(x_7); +x_11 = l_Lean_Elab_elabModifiers___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_9, x_10, x_8); lean_dec(x_3); lean_dec(x_2); -return x_10; +return x_11; } } LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__2___boxed(lean_object** _args) { @@ -3154,16 +3170,17 @@ lean_object* x_14 = _args[13]; lean_object* x_15 = _args[14]; lean_object* x_16 = _args[15]; lean_object* x_17 = _args[16]; +lean_object* x_18 = _args[17]; _start: { -uint8_t x_18; uint8_t x_19; lean_object* x_20; -x_18 = lean_unbox(x_5); -lean_dec(x_5); -x_19 = lean_unbox(x_17); -lean_dec(x_17); -x_20 = l_Lean_Elab_elabModifiers___rarg___lambda__2(x_1, x_2, x_3, x_4, x_18, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_19); +uint8_t x_19; uint8_t x_20; lean_object* x_21; +x_19 = lean_unbox(x_6); lean_dec(x_6); -return x_20; +x_20 = lean_unbox(x_18); +lean_dec(x_18); +x_21 = l_Lean_Elab_elabModifiers___rarg___lambda__2(x_1, x_2, x_3, x_4, x_5, x_19, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_20); +lean_dec(x_7); +return x_21; } } LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__3___boxed(lean_object** _args) { @@ -3184,23 +3201,15 @@ lean_object* x_14 = _args[13]; lean_object* x_15 = _args[14]; lean_object* x_16 = _args[15]; lean_object* x_17 = _args[16]; +lean_object* x_18 = _args[17]; _start: { -uint8_t x_18; lean_object* x_19; -x_18 = lean_unbox(x_4); -lean_dec(x_4); -x_19 = l_Lean_Elab_elabModifiers___rarg___lambda__3(x_1, x_2, x_3, x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); -lean_dec(x_16); -return x_19; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -lean_object* x_13; -x_13 = l_Lean_Elab_elabModifiers___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_12); -return x_13; +uint8_t x_19; lean_object* x_20; +x_19 = lean_unbox(x_5); +lean_dec(x_5); +x_20 = l_Lean_Elab_elabModifiers___rarg___lambda__3(x_1, x_2, x_3, x_4, x_19, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18); +lean_dec(x_17); +return x_20; } } LEAN_EXPORT lean_object* l_Lean_Elab_applyVisibility___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { @@ -3919,7 +3928,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_mkDeclName___rarg___lambda__3(lean_object* _start: { uint8_t x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_11 = lean_ctor_get_uint8(x_1, sizeof(void*)*2); +x_11 = lean_ctor_get_uint8(x_1, sizeof(void*)*3); lean_inc(x_4); lean_inc(x_2); x_12 = l_Lean_Elab_applyVisibility___rarg(x_2, x_3, x_4, x_5, x_11, x_6); @@ -4478,7 +4487,7 @@ lean_inc(x_8); x_9 = lean_ctor_get(x_7, 1); lean_inc(x_9); lean_dec(x_7); -x_10 = lean_ctor_get(x_1, 0); +x_10 = lean_ctor_get(x_1, 1); lean_inc(x_10); lean_dec(x_1); lean_inc(x_8); diff --git a/stage0/stdlib/Lean/Elab/Declaration.c b/stage0/stdlib/Lean/Elab/Declaration.c index d821ce959d6e..bca92a28e7ef 100644 --- a/stage0/stdlib/Lean/Elab/Declaration.c +++ b/stage0/stdlib/Lean/Elab/Declaration.c @@ -18,23 +18,20 @@ lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabAxiom___lambda__4___closed__2; lean_object* l_Lean_Elab_Term_levelMVarToParam(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -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*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabMutual__1(lean_object*); lean_object* lean_format_pretty(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__8; static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__37; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInitialize___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_setDefName___closed__3; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__8; static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__29; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAttr(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualElement__1___closed__2; lean_object* l_Lean_MapDeclarationExtension_insert___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__3; static lean_object* l_Lean_Elab_Command_elabAxiom___lambda__4___closed__9; lean_object* l_Lean_Attribute_erase(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t l_Lean_Elab_Command_isMutualInductive(lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isInstanceDef(lean_object*); static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_setDeclIdName___closed__2; @@ -44,33 +41,24 @@ static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__35; static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__47; static lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclaration_declRange__1___closed__2; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_ensureValidNamespace___closed__3; -lean_object* l_Lean_addDocString_x27___at_Lean_Elab_Command_expandDeclId___spec__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualNamespace__1___closed__5; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandMutualElement___spec__1___lambda__1___boxed(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___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___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*); static lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabAttr___spec__5___closed__4; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualNamespace__1(lean_object*); lean_object* l_Lean_Elab_Command_runTermElabM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_sortDeclLevelParams(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*); static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualPreambleCommand___closed__9; extern lean_object* l_Lean_declRangeExt; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabAttr__1(lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclaration__1(lean_object*); static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualPreambleCommand___closed__7; -static lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__3___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualNamespace__1___closed__2; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_ensureValidNamespace___closed__4; -lean_object* l_Lean_Elab_Command_getLevelNames___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandMutualPreamble(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getHeadInfo(lean_object*); @@ -84,35 +72,29 @@ static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__20; static lean_object* l_Lean_Elab_Command_expandMutualElement___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1___closed__1; lean_object* l_Lean_FileMap_toPosition(lean_object*, 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_Lean_Elab_Command_elabInitialize___lambda__1___closed__49; static lean_object* l_Lean_Elab_Command_expandMutualPreamble___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualPreamble_declRange__1___closed__7; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_Command_expandMutualNamespace___spec__2(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandMutualElement___spec__1___lambda__1(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_toString(lean_object*, uint8_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__13; lean_object* l_Lean_Syntax_getId(lean_object*); -static lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__1___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Command_elabInitialize___spec__1___closed__2; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_ensureValidNamespace___closed__1; -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_expandMutualNamespace___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_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*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualElement_declRange__1___closed__5; -LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabAttr__1___closed__3; lean_object* lean_array_push(lean_object*, lean_object*); lean_object* l_Array_toSubarray___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__6(lean_object*, size_t, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualInductive___boxed(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabAttr__1___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_expandNamespacedDeclaration__1(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInductive(lean_object*, lean_object*, 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__1; +lean_object* l_Lean_Elab_Command_elabInductive(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_mk_array(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isInstanceDef___closed__1; static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__6___closed__4; @@ -122,33 +104,27 @@ static lean_object* l_Lean_Elab_Command_elabAxiom___lambda__4___closed__7; extern lean_object* l_Lean_Elab_Term_instMonadTermElabM; lean_object* l_Lean_Syntax_getArgs(lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__3___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___at_Lean_Elab_Command_elabInitialize___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_compileDecl(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_replaceRef(lean_object*, lean_object*); lean_object* l_instInhabitedReaderT___rarg___boxed(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandNamespacedDeclaration_declRange__1___closed__6; static lean_object* l_Lean_Elab_Command_elabAxiom___lambda__4___closed__11; +lean_object* l_Lean_Elab_Command_elabMutualInductive(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_inductiveSyntaxToView___closed__4; -lean_object* l_Lean_Syntax_getPos_x3f(lean_object*, uint8_t); lean_object* l_Lean_Elab_Command_elabCommand(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandNamespacedDeclaration_declRange__1___closed__7; -static lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__6; -lean_object* l_Lean_Syntax_getTailPos_x3f(lean_object*, uint8_t); static lean_object* l___regBuiltin_Lean_Elab_Command_elabAttr__1___closed__4; -static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__3___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabDeclaration___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabInitialize___spec__4___closed__1; lean_object* l_Lean_Macro_throwError___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabDeclaration___closed__1; static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__17; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualPreamble_declRange__1___closed__1; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__9; -LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_elabMutualInductive(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Command_elabInitialize___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInitialize___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_elabClassInductive___closed__3; -lean_object* l_Lean_Syntax_getIdAt(lean_object*, lean_object*); lean_object* l_Lean_logAt___at_Lean_Elab_Command_runLinters___spec__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__6; lean_object* l_Lean_addBuiltinDeclarationRanges(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkIdentFrom(lean_object*, lean_object*, uint8_t); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__13; @@ -157,7 +133,6 @@ static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualPreamble__1___c LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualElement_declRange__1(lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualPreambleCommand(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1___closed__5; -uint8_t l_Lean_Linter_getLinterValue(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__2; lean_object* l_Lean_Syntax_node5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabAttr__1___closed__1; @@ -171,35 +146,30 @@ static lean_object* l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1___clo lean_object* l_EStateM_instMonad(lean_object*, lean_object*); uint8_t l_Lean_MapDeclarationExtension_contains___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInitialize(lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_List_head_x21___rarg(lean_object*, lean_object*); -lean_object* l_Lean_Elab_applyVisibility___at_Lean_Elab_Command_expandDeclId___spec__6(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_string_dec_eq(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabMutual_declRange__1___closed__4; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__20; static lean_object* l_Lean_Elab_Command_elabInitialize___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualPreamble__1___closed__1; static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__2___closed__3; -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*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_ensureValidNamespace___lambda__2___boxed(lean_object*); uint8_t l_Lean_Name_isPrefixOf(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabMutual_declRange__1___closed__5; static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__2___closed__4; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__7; -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*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Command_expandNamespacedDeclaration__1___closed__2; lean_object* l_Lean_CollectLevelParams_main(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__6; -lean_object* l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__25; static lean_object* l_Lean_ensureNonAmbiguous___at_Lean_Elab_Command_elabAttr___spec__2___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Command_elabInitialize___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_withSaveInfoContext___at___private_Lean_Elab_PreDefinition_Basic_0__Lean_Elab_addNonRecAux___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___closed__1; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__5; lean_object* l_Lean_Elab_Command_withoutCommandIncrementality___rarg(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualNamespace_declRange__1___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Command_elabMutual__1___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; lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Doc_elabTacticExtension___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabMutual_declRange__1___closed__7; static lean_object* l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; @@ -207,19 +177,16 @@ static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualPreamble_declRa lean_object* l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___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*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualNamespace_declRange__1___closed__5; static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualElement__1___closed__1; -lean_object* l_Lean_Elab_Modifiers_addAttr(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabDeclaration___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabInitialize___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__8; static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__28; size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInitialize___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabMutual__2(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isInstanceDef___boxed(lean_object*); -static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabDeclaration___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__21; LEAN_EXPORT uint8_t l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_ensureValidNamespace___lambda__2(lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__3; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabAttr___spec__5___closed__1; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__6; static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualElement__1___closed__3; @@ -230,14 +197,13 @@ static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__30; static lean_object* l_Lean_Elab_Command_expandNamespacedDeclaration___closed__6; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__1; extern lean_object* l_Lean_Elab_Command_commandElabAttribute; -LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualPreamble__1(lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__43; static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__3___closed__6; static lean_object* l_Lean_ensureNonAmbiguous___at_Lean_Elab_Command_elabAttr___spec__2___closed__5; +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Command_elabInitialize___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_getDeclarationSelectionRef(lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__5; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabMutual_declRange__1___closed__1; lean_object* l_Lean_mkPrivateName(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__13; @@ -246,15 +212,12 @@ static lean_object* l_Lean_Elab_Command_elabAttr___closed__1; static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__19; lean_object* l_Lean_SourceInfo_fromRef(lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInitialize___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -uint8_t l_Lean_Elab_Modifiers_isProtected(lean_object*); -LEAN_EXPORT uint8_t l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualInductive(lean_object*); lean_object* l_Lean_Syntax_node6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__12; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_expandMutualNamespace___spec__3(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef(lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__6___closed__1; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__4; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_elabMutualInductive___spec__1(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualElement_declRange__1___closed__1; lean_object* l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__16; @@ -266,31 +229,26 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_ lean_object* l_Lean_Elab_Command_getRef(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__6___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Command_findCommonPrefix_findCommon(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__4; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualPreambleCommand___closed__4; 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_object* l_Lean_Name_components(lean_object*); lean_object* l_Lean_Syntax_getKind(lean_object*); -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_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__3___closed__2; lean_object* l_Lean_MessageData_ofFormat(lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__6___closed__5; static lean_object* l_Lean_ensureNonAmbiguous___at_Lean_Elab_Command_elabAttr___spec__2___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabDeclaration___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualNamespace_declRange__1___closed__2; -static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___closed__2; lean_object* l_Lean_Elab_elabAttrs___at_Lean_Elab_Command_elabMutualDef___spec__3(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* l_Lean_Name_replacePrefix(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabDeclaration___closed__3; +lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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_st_ref_get(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__38; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__2; lean_object* l_Lean_Elab_addBuiltinIncrementalElab(lean_object*, lean_object*); uint8_t l_Lean_Elab_Command_isDefLike(lean_object*); lean_object* l_Lean_Syntax_getOptional_x3f(lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__5; lean_object* lean_array_to_list(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualElement_declRange__1___closed__7; LEAN_EXPORT lean_object* l_Lean_Elab_Command_findCommonPrefix_findCommon___boxed(lean_object*, lean_object*); @@ -305,10 +263,8 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInitialize___lambda__2___boxed( LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabMutual_declRange__1___closed__6; lean_object* l_Lean_Name_append(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Command_elabAxiom___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Command_elabAxiom___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__4; static lean_object* l___regBuiltin_Lean_Elab_Command_elabMutual_declRange__1___closed__3; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__12; static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualPreamble_declRange__1___closed__3; static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__6___closed__2; lean_object* l_Lean_Elab_expandDeclSig(lean_object*); @@ -316,33 +272,30 @@ static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__9; static lean_object* l_Lean_Elab_Command_elabInitialize___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabDeclaration___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_setDeclIdName___closed__3; -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualInductive___spec__1___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__4; -static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__11; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInitialize___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Command_getCurrMacroScope(lean_object*, lean_object*, lean_object*); -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*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabDeclaration___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_expandDeclIdCore(lean_object*); lean_object* l_Lean_Syntax_getSepArgs(lean_object*); lean_object* l_Lean_addMacroScope(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___closed__1; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__3; static lean_object* l_Lean_Elab_Command_elabAxiom___lambda__4___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAttr___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__4; lean_object* l_Lean_extractMacroScopes(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandNamespacedDeclaration_declRange__1___closed__3; -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*); uint8_t lean_name_eq(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_setDeclIdName___closed__1; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabAxiom___lambda__4___closed__10; +lean_object* l_Lean_Elab_Term_getLevelNames___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__3___closed__2; static lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabAttr___spec__5___closed__2; extern lean_object* l_Lean_Elab_macroAttribute; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__18; uint8_t l_Lean_isExtern(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___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_throwErrorAt___at_Lean_Elab_Term_processDefDeriving___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_node2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualDef(lean_object*); @@ -355,59 +308,54 @@ static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNam lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_expandMutualNamespace___spec__3___closed__1; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__10; uint8_t l_Lean_Syntax_matchesNull(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__6___lambda__1(lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__12; static lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclaration__1___closed__4; 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*); uint8_t l_Lean_Syntax_isIdent(lean_object*); static lean_object* l_Lean_Elab_Command_elabMutual___closed__2; 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*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__40; -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*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualElement__1(lean_object*); lean_object* lean_mk_syntax_ident(lean_object*); static lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabAttr___spec__5___closed__3; lean_object* l_Lean_Elab_Command_getScope___rarg(lean_object*, lean_object*); -lean_object* l_Lean_TSyntax_getDocString(lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__2___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Command_expandNamespacedDeclaration_declRange__1___closed__4; -static lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__2; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__10; +lean_object* l_Lean_Elab_Term_withAutoBoundImplicitForbiddenPred___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Std_Format_defWidth; static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualPreamble_declRange__1___closed__5; lean_object* l_Lean_MacroScopesView_review(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualElement_declRange__1___closed__3; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_expandMutualNamespace___spec__3___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310_(lean_object*); lean_object* l_Lean_Elab_realizeGlobalConstWithInfos(lean_object*, lean_object*, lean_object*, lean_object*, 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_Command_elabClassInductive(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualNamespace__1___closed__4; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___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*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__39; static lean_object* l_panic___at_Lean_Elab_Command_expandMutualNamespace___spec__2___closed__1; static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__15; -static lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__1; -static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__5; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualPreambleCommand___closed__5; lean_object* l_Array_append___rarg(lean_object*, lean_object*); -lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofExpr(lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__13; static lean_object* l_Lean_ensureNonAmbiguous___at_Lean_Elab_Command_elabAttr___spec__2___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Command_elabInitialize__1___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_splitMutualPreamble_loop(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_splitMutualPreamble(lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__10; lean_object* l_panic___at_Lean_Parser_SyntaxStack_back___spec__1(lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__2; lean_object* l_Lean_Syntax_node4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_setDeclIdName___closed__4; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_elabMutualInductive___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualElement_declRange__1___closed__6; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__16; static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__46; static lean_object* l_Lean_Elab_Command_elabAxiom___lambda__4___closed__5; static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualPreamble__1___closed__3; lean_object* l_Lean_Syntax_setArg(lean_object*, lean_object*, lean_object*); -uint8_t l_Lean_Elab_Modifiers_isPrivate(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_setDefName(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___closed__1; lean_object* l_Lean_Elab_Term_addTermInfo_x27(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -415,25 +363,21 @@ static lean_object* l___regBuiltin_Lean_Elab_Command_expandNamespacedDeclaration lean_object* l_Lean_FileMap_leanPosToLspPos(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_expandNamespacedDeclaration___closed__3; uint8_t l_Lean_Syntax_isToken(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_classInductiveSyntaxToView(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_ensureValidNamespace___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__6___closed__3; static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__33; static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__32; +lean_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___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualPreambleCommand___boxed(lean_object*); -lean_object* l_Lean_Elab_getOptDerivingClasses(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__9; static lean_object* l_Lean_Elab_Command_expandMutualPreamble___closed__3; -static lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__3; -static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__3___closed__2; LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualDef___spec__1(lean_object*, size_t, size_t); -static lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__2___closed__1; static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__3___closed__4; static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__26; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_expandMutualNamespace___spec__3___closed__2; static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__11; lean_object* l_Lean_Meta_Simp_isBuiltinSimproc(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_elabClassInductive___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandMutualPreamble___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__41; uint8_t lean_nat_dec_eq(lean_object*, lean_object*); @@ -442,40 +386,33 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabDeclaration(lean_object*, lean_ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclaration__2(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualDef___spec__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabInitialize__1(lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__11; -static lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandMutualNamespace(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInitialize___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Name_beq___boxed(lean_object*, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandNamespacedDeclaration(lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualNamespace_declRange__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___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_Elab_Command_elabMutualDef(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__4(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_expandMutualElement___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_expandNamespacedDeclaration___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualNamespace__1___closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__31; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_elabBinders___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__3___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Elab_Command_elabInductiveViews(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualElement_declRange__1___closed__4; -LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_setDeclIdName___closed__6; uint8_t l_Lean_isAttribute(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_elabInitialize___lambda__3___closed__5; +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Command_elabInitialize___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabAxiom___lambda__4___closed__8; -LEAN_EXPORT lean_object* l_Lean_Linter_logLintIf___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabMutual__1___closed__3; 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_object* l_Lean_Syntax_node1(lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclaration__1___closed__3; 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_Lean_Elab_Term_expandDeclId(lean_object*, lean_object*, 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_elabAxiom___lambda__4___closed__1; static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__6___closed__7; static lean_object* l_Lean_Elab_Command_expandMutualPreamble___closed__2; @@ -490,11 +427,7 @@ static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNam static lean_object* l_Lean_Elab_Command_elabDeclaration___closed__2; 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_object* l_Lean_throwError___at___private_Lean_Elab_Command_0__Lean_Elab_Command_elabCommandUsing___spec__1___boxed(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*); static lean_object* l_Lean_ensureNonAmbiguous___at_Lean_Elab_Command_elabAttr___spec__2___closed__4; -LEAN_EXPORT lean_object* l_Lean_Linter_logLintIf___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__7; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualNamespace_declRange__1___closed__1; lean_object* l_Lean_Syntax_setInfo(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclaration_declRange__1___closed__3; @@ -503,14 +436,11 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAtt static lean_object* l_Lean_Elab_Command_expandNamespacedDeclaration___closed__1; lean_object* l_Array_mkArray1___rarg(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Elab_Command_liftCoreM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Syntax_getRange_x3f(lean_object*, uint8_t); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__24; -static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__2___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_findCommonPrefix(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandNamespacedDeclaration_docString__1___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclaration_declRange__1___closed__1; -lean_object* l_Lean_Elab_expandOptDeclSig(lean_object*); -extern lean_object* l_Lean_Linter_linter_deprecated; lean_object* l_Array_ofSubarray___rarg(lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__3___closed__7; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -523,12 +453,11 @@ LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_Command_elabAttr___spec__3(lean_ static lean_object* l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1___closed__3; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__11; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isInstanceDef___closed__2; -extern lean_object* l_Lean_Elab_Command_instInhabitedScope; lean_object* lean_array_mk(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclaration__1___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__6___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__6; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Command_elabInitialize___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabAttr__1___closed__5; static lean_object* l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1___closed__6; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__1; @@ -538,39 +467,36 @@ static lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclaration_declRange__ size_t lean_usize_add(size_t, size_t); static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__8; lean_object* l_List_mapTR_loop___at_Lean_ensureNonAmbiguous___spec__2(lean_object*, lean_object*); -lean_object* l_Lean_Elab_Command_expandDeclId(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabAxiom___lambda__4___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclaration_declRange__1___closed__6; static lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclaration__1___closed__2; lean_object* l_Lean_Macro_expandMacro_x3f(lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_instInhabitedName; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); 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_throwUnknownConstant___at_Lean_Elab_Command_elabAttr___spec__5___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); size_t lean_array_size(lean_object*); static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__4; -LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_expandNamespacedDeclaration_declRange__1(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandNamespacedDeclaration__1___closed__4; +static lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Command_elabInitialize___spec__1___closed__1; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualPreambleCommand___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024_(lean_object*); lean_object* l_instInhabitedOfMonad___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_ensureValidNamespace___boxed(lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_instInhabitedSyntax; lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Command_elabInitialize___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabMutual(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclaration_declRange__1___closed__4; -static lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___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_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_ensureValidNamespace___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualPreambleCommand___closed__8; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__2; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_setDefName___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandMutualElement(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__42; -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*); static lean_object* l_Lean_Elab_Command_elabAxiom___lambda__4___closed__3; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_setDefName___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabDeclaration___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -581,26 +507,25 @@ static lean_object* l___regBuiltin_Lean_Elab_Command_expandNamespacedDeclaration LEAN_EXPORT lean_object* l_Lean_Elab_Command_findCommonPrefix_go(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualPreamble_declRange__1(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualNamespace_declRange__1___closed__7; -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualInductive___spec__1(lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclaration_declRange__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabMutual___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__44; lean_object* lean_array_get_size(lean_object*); LEAN_EXPORT lean_object* l_Lean_ensureNonAmbiguous___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_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabMutual_declRange__1___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_setDeclIdName(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_expandMutualNamespace___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__7; static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___at_Lean_Elab_Command_elabInitialize___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__2___closed__5; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_setDeclIdName___closed__5; static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualElement_declRange__1___closed__2; uint8_t lean_usize_dec_lt(size_t, size_t); -static lean_object* l_Lean_Elab_Command_elabClassInductive___closed__2; lean_object* l_Array_mkArray2___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualNamespace_declRange__1(lean_object*); -static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___closed__3; +LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabInitialize___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandNamespacedDeclaration_declRange__1___closed__1; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Command_expandNamespacedDeclaration_declRange__1___closed__5; @@ -609,7 +534,6 @@ lean_object* lean_nat_add(lean_object*, lean_object*); static lean_object* l_panic___at_Lean_Elab_Command_expandMutualNamespace___spec__2___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInitialize___lambda__6___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_Exception_isRuntime(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabSyntax___spec__1___rarg(lean_object*); static lean_object* l_Lean_Elab_Command_elabMutual___closed__3; lean_object* l_Lean_mkConstWithLevelParams___at_Lean_Elab_Term_expandDeclId___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -629,11 +553,8 @@ lean_object* l_Lean_MessageData_ofName(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualNamespace_declRange__1___closed__6; static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__14; static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__23; -uint8_t l_Lean_Elab_Modifiers_isPartial(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__1; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualPreambleCommand___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabDeclaration___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabInitialize__1___closed__3; lean_object* l_Lean_addDecl(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__10; @@ -1659,4147 +1580,1735 @@ lean_dec(x_2); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Command_elabAxiom___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_5; uint8_t x_6; lean_object* x_7; lean_object* x_8; -x_5 = lean_ctor_get(x_2, 1); -lean_inc(x_5); -lean_dec(x_2); -x_6 = 0; -x_7 = l_Lean_Syntax_getPos_x3f(x_1, x_6); -x_8 = l_Lean_Syntax_getTailPos_x3f(x_1, x_6); -if (lean_obj_tag(x_7) == 0) -{ -lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_9 = lean_unsigned_to_nat(0u); -lean_inc(x_5); -x_10 = l_Lean_FileMap_toPosition(x_5, x_9); -lean_inc(x_10); -x_11 = l_Lean_FileMap_leanPosToLspPos(x_5, x_10); -if (lean_obj_tag(x_8) == 0) -{ -uint8_t x_12; -lean_dec(x_5); -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, 1); -x_14 = lean_ctor_get(x_11, 0); -lean_dec(x_14); -lean_inc(x_13); -lean_inc(x_10); -x_15 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_15, 0, x_10); -lean_ctor_set(x_15, 1, x_13); -lean_ctor_set(x_15, 2, x_10); -lean_ctor_set(x_15, 3, x_13); -lean_ctor_set(x_11, 1, x_4); -lean_ctor_set(x_11, 0, x_15); -return x_11; -} -else -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_11, 1); -lean_inc(x_16); -lean_dec(x_11); -lean_inc(x_16); -lean_inc(x_10); -x_17 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_17, 0, x_10); -lean_ctor_set(x_17, 1, x_16); -lean_ctor_set(x_17, 2, x_10); -lean_ctor_set(x_17, 3, x_16); -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_17); -lean_ctor_set(x_18, 1, x_4); -return x_18; -} -} -else -{ -uint8_t x_19; -x_19 = !lean_is_exclusive(x_11); -if (x_19 == 0) +lean_object* x_10; +lean_inc(x_3); +x_10 = l_Lean_mkConstWithLevelParams___at_Lean_Elab_Term_expandDeclId___spec__7(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_10) == 0) { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_20 = lean_ctor_get(x_11, 1); -x_21 = lean_ctor_get(x_11, 0); -lean_dec(x_21); -x_22 = lean_ctor_get(x_8, 0); -lean_inc(x_22); -lean_dec(x_8); -lean_inc(x_5); -x_23 = l_Lean_FileMap_toPosition(x_5, x_22); -lean_dec(x_22); -lean_inc(x_23); -x_24 = l_Lean_FileMap_leanPosToLspPos(x_5, x_23); -lean_dec(x_5); -x_25 = lean_ctor_get(x_24, 1); -lean_inc(x_25); -lean_dec(x_24); -x_26 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_26, 0, x_10); -lean_ctor_set(x_26, 1, x_20); -lean_ctor_set(x_26, 2, x_23); -lean_ctor_set(x_26, 3, x_25); -lean_ctor_set(x_11, 1, x_4); -lean_ctor_set(x_11, 0, x_26); -return x_11; +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; lean_object* x_16; +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_10, 1); +lean_inc(x_12); +lean_dec(x_10); +x_13 = lean_box(0); +x_14 = lean_box(0); +x_15 = 1; +x_16 = l_Lean_Elab_Term_addTermInfo_x27(x_2, x_11, x_13, x_13, x_14, x_15, x_3, x_4, x_5, x_6, x_7, x_8, x_12); +return x_16; } else { -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_27 = lean_ctor_get(x_11, 1); -lean_inc(x_27); -lean_dec(x_11); -x_28 = lean_ctor_get(x_8, 0); -lean_inc(x_28); +uint8_t x_17; lean_dec(x_8); -lean_inc(x_5); -x_29 = l_Lean_FileMap_toPosition(x_5, x_28); -lean_dec(x_28); -lean_inc(x_29); -x_30 = l_Lean_FileMap_leanPosToLspPos(x_5, x_29); -lean_dec(x_5); -x_31 = lean_ctor_get(x_30, 1); -lean_inc(x_31); -lean_dec(x_30); -x_32 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_32, 0, x_10); -lean_ctor_set(x_32, 1, x_27); -lean_ctor_set(x_32, 2, x_29); -lean_ctor_set(x_32, 3, x_31); -x_33 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_33, 0, x_32); -lean_ctor_set(x_33, 1, x_4); -return x_33; -} -} -} -else -{ -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_7, 0); -lean_inc(x_34); lean_dec(x_7); -lean_inc(x_5); -x_35 = l_Lean_FileMap_toPosition(x_5, x_34); -lean_dec(x_34); -lean_inc(x_35); -x_36 = l_Lean_FileMap_leanPosToLspPos(x_5, x_35); -if (lean_obj_tag(x_8) == 0) -{ -uint8_t x_37; +lean_dec(x_6); lean_dec(x_5); -x_37 = !lean_is_exclusive(x_36); -if (x_37 == 0) -{ -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_36, 1); -x_39 = lean_ctor_get(x_36, 0); -lean_dec(x_39); -lean_inc(x_38); -lean_inc(x_35); -x_40 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_40, 0, x_35); -lean_ctor_set(x_40, 1, x_38); -lean_ctor_set(x_40, 2, x_35); -lean_ctor_set(x_40, 3, x_38); -lean_ctor_set(x_36, 1, x_4); -lean_ctor_set(x_36, 0, x_40); -return x_36; -} -else +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_17 = !lean_is_exclusive(x_10); +if (x_17 == 0) { -lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_ctor_get(x_36, 1); -lean_inc(x_41); -lean_dec(x_36); -lean_inc(x_41); -lean_inc(x_35); -x_42 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_42, 0, x_35); -lean_ctor_set(x_42, 1, x_41); -lean_ctor_set(x_42, 2, x_35); -lean_ctor_set(x_42, 3, x_41); -x_43 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_43, 0, x_42); -lean_ctor_set(x_43, 1, x_4); -return x_43; -} +return x_10; } else { -uint8_t x_44; -x_44 = !lean_is_exclusive(x_36); -if (x_44 == 0) -{ -lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_45 = lean_ctor_get(x_36, 1); -x_46 = lean_ctor_get(x_36, 0); -lean_dec(x_46); -x_47 = lean_ctor_get(x_8, 0); -lean_inc(x_47); -lean_dec(x_8); -lean_inc(x_5); -x_48 = l_Lean_FileMap_toPosition(x_5, x_47); -lean_dec(x_47); -lean_inc(x_48); -x_49 = l_Lean_FileMap_leanPosToLspPos(x_5, x_48); -lean_dec(x_5); -x_50 = lean_ctor_get(x_49, 1); -lean_inc(x_50); -lean_dec(x_49); -x_51 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_51, 0, x_35); -lean_ctor_set(x_51, 1, x_45); -lean_ctor_set(x_51, 2, x_48); -lean_ctor_set(x_51, 3, x_50); -lean_ctor_set(x_36, 1, x_4); -lean_ctor_set(x_36, 0, x_51); -return x_36; +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_10, 0); +x_19 = lean_ctor_get(x_10, 1); +lean_inc(x_19); +lean_inc(x_18); +lean_dec(x_10); +x_20 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_20, 0, x_18); +lean_ctor_set(x_20, 1, x_19); +return x_20; } -else -{ -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; -x_52 = lean_ctor_get(x_36, 1); -lean_inc(x_52); -lean_dec(x_36); -x_53 = lean_ctor_get(x_8, 0); -lean_inc(x_53); -lean_dec(x_8); -lean_inc(x_5); -x_54 = l_Lean_FileMap_toPosition(x_5, x_53); -lean_dec(x_53); -lean_inc(x_54); -x_55 = l_Lean_FileMap_leanPosToLspPos(x_5, x_54); -lean_dec(x_5); -x_56 = lean_ctor_get(x_55, 1); -lean_inc(x_56); -lean_dec(x_55); -x_57 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_57, 0, x_35); -lean_ctor_set(x_57, 1, x_52); -lean_ctor_set(x_57, 2, x_54); -lean_ctor_set(x_57, 3, x_56); -x_58 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_58, 0, x_57); -lean_ctor_set(x_58, 1, x_4); -return x_58; } } } +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___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: +{ +uint8_t x_11; lean_object* x_12; +x_11 = 1; +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); +return x_12; } } -static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__3___closed__1() { +static lean_object* _init_l_Lean_Elab_Command_elabAxiom___lambda__3___closed__1() { _start: { lean_object* x_1; -x_1 = l_Lean_declRangeExt; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_withSaveInfoContext___at___private_Lean_Elab_PreDefinition_Basic_0__Lean_Elab_addNonRecAux___spec__1___lambda__1___boxed), 7, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_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_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_1); +x_13 = l_Lean_Elab_Term_ensureNoUnassignedMVars(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_13) == 0) { -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, 0); -x_9 = lean_ctor_get(x_6, 1); -x_10 = lean_ctor_get(x_8, 0); +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_13, 1); +lean_inc(x_14); +lean_dec(x_13); +lean_inc(x_11); lean_inc(x_10); -lean_dec(x_8); -x_11 = l_Lean_instInhabitedDeclarationRanges; -x_12 = l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__3___closed__1; lean_inc(x_1); -x_13 = l_Lean_MapDeclarationExtension_contains___rarg(x_11, x_12, x_10, x_1); -lean_dec(x_10); -if (x_13 == 0) +x_15 = l_Lean_addDecl(x_1, x_10, x_11, x_14); +if (lean_obj_tag(x_15) == 0) { -lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; -lean_free_object(x_6); -x_14 = lean_st_ref_take(x_4, x_9); -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; +x_16 = lean_ctor_get(x_15, 1); lean_inc(x_16); -lean_dec(x_14); -x_17 = !lean_is_exclusive(x_15); -if (x_17 == 0) +lean_dec(x_15); +lean_inc(x_2); +x_17 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabAxiom___lambda__1), 9, 2); +lean_closure_set(x_17, 0, x_2); +lean_closure_set(x_17, 1, x_3); +x_18 = l_Lean_Elab_Command_elabAxiom___lambda__3___closed__1; +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +x_19 = l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at___private_Lean_Elab_PreDefinition_Basic_0__Lean_Elab_addNonRecAux___spec__2(x_17, x_18, x_6, x_7, x_8, x_9, x_10, x_11, x_16); +if (lean_obj_tag(x_19) == 0) { -lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; -x_18 = lean_ctor_get(x_15, 0); -x_19 = l_Lean_MapDeclarationExtension_insert___rarg(x_12, x_18, x_1, x_2); -lean_ctor_set(x_15, 0, x_19); -x_20 = lean_st_ref_set(x_4, x_15, x_16); -x_21 = !lean_is_exclusive(x_20); -if (x_21 == 0) +lean_object* x_20; uint8_t x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_19, 1); +lean_inc(x_20); +lean_dec(x_19); +x_21 = 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_4); +lean_inc(x_2); +x_22 = l_Lean_Elab_Term_applyAttributesAt(x_2, x_4, x_21, x_6, x_7, x_8, x_9, x_10, x_11, x_20); +if (lean_obj_tag(x_22) == 0) { -lean_object* x_22; lean_object* x_23; -x_22 = lean_ctor_get(x_20, 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; +x_23 = lean_ctor_get(x_22, 1); +lean_inc(x_23); 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; lean_object* x_40; lean_object* x_41; -x_27 = lean_ctor_get(x_15, 0); -x_28 = lean_ctor_get(x_15, 1); -x_29 = lean_ctor_get(x_15, 2); -x_30 = lean_ctor_get(x_15, 3); -x_31 = lean_ctor_get(x_15, 4); -x_32 = lean_ctor_get(x_15, 5); -x_33 = lean_ctor_get(x_15, 6); -x_34 = lean_ctor_get(x_15, 7); -lean_inc(x_34); -lean_inc(x_33); -lean_inc(x_32); -lean_inc(x_31); -lean_inc(x_30); -lean_inc(x_29); -lean_inc(x_28); -lean_inc(x_27); -lean_dec(x_15); -x_35 = l_Lean_MapDeclarationExtension_insert___rarg(x_12, x_27, x_1, x_2); -x_36 = lean_alloc_ctor(0, 8, 0); -lean_ctor_set(x_36, 0, x_35); -lean_ctor_set(x_36, 1, x_28); -lean_ctor_set(x_36, 2, x_29); -lean_ctor_set(x_36, 3, x_30); -lean_ctor_set(x_36, 4, x_31); -lean_ctor_set(x_36, 5, x_32); -lean_ctor_set(x_36, 6, x_33); -lean_ctor_set(x_36, 7, x_34); -x_37 = lean_st_ref_set(x_4, x_36, x_16); -x_38 = lean_ctor_get(x_37, 1); -lean_inc(x_38); -if (lean_is_exclusive(x_37)) { - lean_ctor_release(x_37, 0); - lean_ctor_release(x_37, 1); - x_39 = x_37; -} else { - lean_dec_ref(x_37); - x_39 = lean_box(0); -} -x_40 = lean_box(0); -if (lean_is_scalar(x_39)) { - x_41 = lean_alloc_ctor(0, 2, 0); -} else { - x_41 = x_39; -} -lean_ctor_set(x_41, 0, x_40); -lean_ctor_set(x_41, 1, x_38); -return x_41; -} -} -else -{ -lean_object* x_42; -lean_dec(x_2); -lean_dec(x_1); -x_42 = lean_box(0); -lean_ctor_set(x_6, 0, x_42); -return x_6; -} -} -else -{ -lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; -x_43 = lean_ctor_get(x_6, 0); -x_44 = lean_ctor_get(x_6, 1); -lean_inc(x_44); -lean_inc(x_43); -lean_dec(x_6); -x_45 = lean_ctor_get(x_43, 0); -lean_inc(x_45); -lean_dec(x_43); -x_46 = l_Lean_instInhabitedDeclarationRanges; -x_47 = l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__3___closed__1; -lean_inc(x_1); -x_48 = l_Lean_MapDeclarationExtension_contains___rarg(x_46, x_47, x_45, x_1); -lean_dec(x_45); -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; -x_49 = lean_st_ref_take(x_4, 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 = lean_ctor_get(x_50, 0); -lean_inc(x_52); -x_53 = lean_ctor_get(x_50, 1); -lean_inc(x_53); -x_54 = lean_ctor_get(x_50, 2); -lean_inc(x_54); -x_55 = lean_ctor_get(x_50, 3); -lean_inc(x_55); -x_56 = lean_ctor_get(x_50, 4); -lean_inc(x_56); -x_57 = lean_ctor_get(x_50, 5); -lean_inc(x_57); -x_58 = lean_ctor_get(x_50, 6); -lean_inc(x_58); -x_59 = lean_ctor_get(x_50, 7); -lean_inc(x_59); -if (lean_is_exclusive(x_50)) { - lean_ctor_release(x_50, 0); - lean_ctor_release(x_50, 1); - lean_ctor_release(x_50, 2); - lean_ctor_release(x_50, 3); - lean_ctor_release(x_50, 4); - lean_ctor_release(x_50, 5); - lean_ctor_release(x_50, 6); - lean_ctor_release(x_50, 7); - x_60 = x_50; -} else { - lean_dec_ref(x_50); - x_60 = lean_box(0); -} -x_61 = l_Lean_MapDeclarationExtension_insert___rarg(x_47, x_52, x_1, x_2); -if (lean_is_scalar(x_60)) { - x_62 = lean_alloc_ctor(0, 8, 0); -} else { - x_62 = x_60; -} -lean_ctor_set(x_62, 0, x_61); -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_56); -lean_ctor_set(x_62, 5, x_57); -lean_ctor_set(x_62, 6, x_58); -lean_ctor_set(x_62, 7, x_59); -x_63 = lean_st_ref_set(x_4, x_62, x_51); -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_box(0); -if (lean_is_scalar(x_65)) { - x_67 = lean_alloc_ctor(0, 2, 0); -} else { - x_67 = x_65; -} -lean_ctor_set(x_67, 0, x_66); -lean_ctor_set(x_67, 1, x_64); -return x_67; -} -else -{ -lean_object* x_68; lean_object* x_69; -lean_dec(x_2); -lean_dec(x_1); -x_68 = lean_box(0); -x_69 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_69, 0, x_68); -lean_ctor_set(x_69, 1, x_44); -return x_69; -} -} -} -} -static lean_object* _init_l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("example", 7, 7); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__1; -x_2 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__2; -x_3 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__3; -x_4 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___closed__1; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; lean_object* x_7; uint8_t x_8; -lean_inc(x_2); -x_6 = l_Lean_Syntax_getKind(x_2); -x_7 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___closed__2; -x_8 = lean_name_eq(x_6, x_7); -lean_dec(x_6); -if (x_8 == 0) -{ -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; -lean_inc(x_3); -x_9 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Command_elabAxiom___spec__2(x_2, x_3, x_4, x_5); -x_10 = lean_ctor_get(x_9, 0); -lean_inc(x_10); -x_11 = lean_ctor_get(x_9, 1); -lean_inc(x_11); -lean_dec(x_9); -x_12 = l_Lean_Elab_getDeclarationSelectionRef(x_2); -lean_inc(x_3); -x_13 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Command_elabAxiom___spec__2(x_12, x_3, x_4, x_11); -lean_dec(x_12); -x_14 = !lean_is_exclusive(x_13); -if (x_14 == 0) -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = lean_ctor_get(x_13, 0); -x_16 = lean_ctor_get(x_13, 1); -lean_ctor_set(x_13, 1, x_15); -lean_ctor_set(x_13, 0, x_10); -x_17 = l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__3(x_1, x_13, x_3, x_4, x_16); -lean_dec(x_3); -return x_17; -} -else -{ -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_18 = lean_ctor_get(x_13, 0); -x_19 = lean_ctor_get(x_13, 1); -lean_inc(x_19); -lean_inc(x_18); -lean_dec(x_13); -x_20 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_20, 0, x_10); -lean_ctor_set(x_20, 1, x_18); -x_21 = l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__3(x_1, x_20, x_3, x_4, x_19); -lean_dec(x_3); -return x_21; -} -} -else -{ -lean_object* x_22; lean_object* x_23; -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_22 = lean_box(0); -x_23 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_23, 0, x_22); -lean_ctor_set(x_23, 1, x_5); -return x_23; -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; -lean_inc(x_3); -x_10 = l_Lean_mkConstWithLevelParams___at_Lean_Elab_Term_expandDeclId___spec__7(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_10) == 0) -{ -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; lean_object* x_16; -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -x_12 = lean_ctor_get(x_10, 1); -lean_inc(x_12); -lean_dec(x_10); -x_13 = lean_box(0); -x_14 = lean_box(0); -x_15 = 1; -x_16 = l_Lean_Elab_Term_addTermInfo_x27(x_2, x_11, x_13, x_13, x_14, x_15, x_3, x_4, x_5, x_6, x_7, x_8, x_12); -return x_16; -} -else -{ -uint8_t x_17; -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_17 = !lean_is_exclusive(x_10); -if (x_17 == 0) -{ -return x_10; -} -else -{ -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_10, 0); -x_19 = lean_ctor_get(x_10, 1); -lean_inc(x_19); -lean_inc(x_18); -lean_dec(x_10); -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_Elab_Command_elabAxiom___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: -{ -uint8_t x_11; lean_object* x_12; -x_11 = 1; -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); -return x_12; -} -} -static lean_object* _init_l_Lean_Elab_Command_elabAxiom___lambda__3___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_withSaveInfoContext___at___private_Lean_Elab_PreDefinition_Basic_0__Lean_Elab_addNonRecAux___spec__1___lambda__1___boxed), 7, 0); -return x_1; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -lean_object* x_13; -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_1); -x_13 = l_Lean_Elab_Term_ensureNoUnassignedMVars(x_1, 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; -x_14 = lean_ctor_get(x_13, 1); -lean_inc(x_14); -lean_dec(x_13); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_1); -x_15 = l_Lean_addDecl(x_1, x_10, x_11, x_14); -if (lean_obj_tag(x_15) == 0) -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_16 = lean_ctor_get(x_15, 1); -lean_inc(x_16); -lean_dec(x_15); -lean_inc(x_2); -x_17 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabAxiom___lambda__1), 9, 2); -lean_closure_set(x_17, 0, x_2); -lean_closure_set(x_17, 1, x_3); -x_18 = l_Lean_Elab_Command_elabAxiom___lambda__3___closed__1; -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -x_19 = l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at___private_Lean_Elab_PreDefinition_Basic_0__Lean_Elab_addNonRecAux___spec__2(x_17, x_18, x_6, x_7, x_8, x_9, x_10, x_11, x_16); -if (lean_obj_tag(x_19) == 0) -{ -lean_object* x_20; uint8_t x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_19, 1); -lean_inc(x_20); -lean_dec(x_19); -x_21 = 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_4); -lean_inc(x_2); -x_22 = l_Lean_Elab_Term_applyAttributesAt(x_2, x_4, x_21, x_6, x_7, x_8, x_9, x_10, x_11, x_20); -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; uint8_t x_28; -x_23 = lean_ctor_get(x_22, 1); -lean_inc(x_23); -lean_dec(x_22); -x_24 = lean_st_ref_get(x_11, x_23); -x_25 = lean_ctor_get(x_24, 0); -lean_inc(x_25); -x_26 = lean_ctor_get(x_24, 1); -lean_inc(x_26); -lean_dec(x_24); -x_27 = lean_ctor_get(x_25, 0); -lean_inc(x_27); -lean_dec(x_25); -lean_inc(x_2); -x_28 = l_Lean_isExtern(x_27, x_2); -lean_dec(x_27); -if (x_28 == 0) -{ -uint8_t x_29; lean_object* x_30; -lean_dec(x_1); -x_29 = 1; -x_30 = l_Lean_Elab_Term_applyAttributesAt(x_2, x_4, x_29, x_6, x_7, x_8, x_9, x_10, x_11, x_26); -return x_30; -} -else -{ -lean_object* x_31; -lean_inc(x_11); -lean_inc(x_10); -x_31 = l_Lean_compileDecl(x_1, x_10, x_11, x_26); -if (lean_obj_tag(x_31) == 0) -{ -lean_object* x_32; uint8_t x_33; lean_object* x_34; -x_32 = lean_ctor_get(x_31, 1); -lean_inc(x_32); -lean_dec(x_31); -x_33 = 1; -x_34 = l_Lean_Elab_Term_applyAttributesAt(x_2, x_4, x_33, x_6, x_7, x_8, x_9, x_10, x_11, x_32); -return x_34; -} -else -{ -uint8_t x_35; -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_4); -lean_dec(x_2); -x_35 = !lean_is_exclusive(x_31); -if (x_35 == 0) -{ -return x_31; -} -else -{ -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; -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -x_39 = !lean_is_exclusive(x_22); -if (x_39 == 0) -{ -return x_22; -} -else -{ -lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_40 = lean_ctor_get(x_22, 0); -x_41 = lean_ctor_get(x_22, 1); -lean_inc(x_41); -lean_inc(x_40); -lean_dec(x_22); -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_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -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_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_47 = !lean_is_exclusive(x_15); -if (x_47 == 0) -{ -return x_15; -} -else -{ -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_51; -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_51 = !lean_is_exclusive(x_13); -if (x_51 == 0) -{ -return x_13; -} -else -{ -lean_object* x_52; lean_object* x_53; lean_object* x_54; -x_52 = lean_ctor_get(x_13, 0); -x_53 = lean_ctor_get(x_13, 1); -lean_inc(x_53); -lean_inc(x_52); -lean_dec(x_13); -x_54 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_54, 0, x_52); -lean_ctor_set(x_54, 1, x_53); -return x_54; -} -} -} -} -static lean_object* _init_l_Lean_Elab_Command_elabAxiom___lambda__4___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(10u); -x_2 = lean_unsigned_to_nat(1u); -x_3 = l_Nat_nextPowerOfTwo_go(x_1, x_2, lean_box(0)); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Command_elabAxiom___lambda__4___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__1; -x_3 = lean_mk_array(x_2, x_1); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Command_elabAxiom___lambda__4___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(0u); -x_2 = l_Lean_Elab_Command_elabAxiom___lambda__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_Elab_Command_elabAxiom___lambda__4___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = lean_box(0); -x_2 = lean_array_mk(x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Elab_Command_elabAxiom___lambda__4___closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__3; -x_2 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__4; -x_3 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_1); -lean_ctor_set(x_3, 2, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Command_elabAxiom___lambda__4___closed__6() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Elab", 4, 4); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Command_elabAxiom___lambda__4___closed__7() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__6; -x_2 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__14; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Command_elabAxiom___lambda__4___closed__8() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("", 0, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Command_elabAxiom___lambda__4___closed__9() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__8; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Elab_Command_elabAxiom___lambda__4___closed__10() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked(" : ", 3, 3); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Command_elabAxiom___lambda__4___closed__11() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__10; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: -{ -lean_object* x_17; uint8_t x_18; lean_object* x_19; -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_17); -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); -if (lean_obj_tag(x_19) == 0) -{ -lean_object* x_20; lean_object* x_21; -x_20 = lean_ctor_get(x_19, 1); -lean_inc(x_20); -lean_dec(x_19); -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_21 = l_Lean_Elab_Term_elabType(x_3, x_10, x_11, x_12, x_13, x_14, x_15, x_20); -if (lean_obj_tag(x_21) == 0) -{ -lean_object* x_22; lean_object* x_23; uint8_t 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 = 1; -x_25 = 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_26 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_24, x_25, x_10, x_11, x_12, x_13, x_14, x_15, x_23); -if (lean_obj_tag(x_26) == 0) -{ -lean_object* x_27; lean_object* x_28; uint8_t x_29; -x_27 = lean_ctor_get(x_26, 1); -lean_inc(x_27); -lean_dec(x_26); -x_28 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_22, x_10, x_11, x_12, x_13, x_14, x_15, x_27); -x_29 = !lean_is_exclusive(x_28); -if (x_29 == 0) -{ -lean_object* x_30; lean_object* x_31; uint8_t x_32; uint8_t x_33; lean_object* x_34; -x_30 = lean_ctor_get(x_28, 0); -x_31 = lean_ctor_get(x_28, 1); -x_32 = 1; -x_33 = 1; -x_34 = l_Lean_Meta_mkForallFVars(x_9, x_30, x_25, x_32, x_33, x_12, x_13, x_14, x_15, x_31); -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); -x_37 = l_Lean_Meta_mkForallFVars(x_4, x_35, x_32, x_32, x_33, x_12, x_13, x_14, x_15, x_36); -if (lean_obj_tag(x_37) == 0) -{ -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_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_Declaration_0__Lean_Elab_Command_ensureValidNamespace___closed__2; -x_41 = l_Lean_Elab_Term_levelMVarToParam(x_38, x_40, x_10, x_11, x_12, x_13, x_14, x_15, x_39); -x_42 = !lean_is_exclusive(x_41); -if (x_42 == 0) -{ -lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; -x_43 = lean_ctor_get(x_41, 0); -x_44 = lean_ctor_get(x_41, 1); -x_45 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__5; -lean_inc(x_43); -x_46 = l_Lean_CollectLevelParams_main(x_43, x_45); -x_47 = lean_ctor_get(x_46, 2); -lean_inc(x_47); -lean_dec(x_46); -x_48 = l_Lean_Elab_sortDeclLevelParams(x_5, x_6, x_47); -if (lean_obj_tag(x_48) == 0) -{ -uint8_t x_49; -lean_free_object(x_41); -lean_dec(x_43); -lean_free_object(x_28); -lean_dec(x_17); -lean_dec(x_8); -lean_dec(x_2); -lean_dec(x_1); -x_49 = !lean_is_exclusive(x_48); -if (x_49 == 0) -{ -lean_object* x_50; lean_object* x_51; -lean_ctor_set_tag(x_48, 3); -x_50 = l_Lean_MessageData_ofFormat(x_48); -x_51 = l_Lean_throwErrorAt___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__12(x_7, x_50, x_10, x_11, x_12, x_13, x_14, x_15, x_44); -lean_dec(x_15); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -return x_51; -} -else -{ -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_52 = lean_ctor_get(x_48, 0); -lean_inc(x_52); -lean_dec(x_48); -x_53 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_53, 0, x_52); -x_54 = l_Lean_MessageData_ofFormat(x_53); -x_55 = l_Lean_throwErrorAt___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__12(x_7, x_54, x_10, x_11, x_12, x_13, x_14, x_15, x_44); -lean_dec(x_15); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -return x_55; -} -} -else -{ -uint8_t x_56; -x_56 = !lean_is_exclusive(x_48); -if (x_56 == 0) -{ -lean_object* x_57; lean_object* x_58; uint8_t x_59; -x_57 = lean_ctor_get(x_48, 0); -x_58 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_43, x_10, x_11, x_12, x_13, x_14, x_15, x_44); -x_59 = !lean_is_exclusive(x_58); -if (x_59 == 0) -{ -lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; uint8_t x_68; -x_60 = lean_ctor_get(x_58, 0); -x_61 = lean_ctor_get(x_58, 1); -lean_inc(x_60); -lean_inc(x_2); -x_62 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_62, 0, x_2); -lean_ctor_set(x_62, 1, x_57); -lean_ctor_set(x_62, 2, x_60); -x_63 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 3); -lean_dec(x_1); -x_64 = lean_alloc_ctor(0, 1, 1); -lean_ctor_set(x_64, 0, x_62); -lean_ctor_set_uint8(x_64, sizeof(void*)*1, x_63); -lean_ctor_set_tag(x_48, 0); -lean_ctor_set(x_48, 0, x_64); -x_65 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__7; -x_66 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_65, x_10, x_11, x_12, x_13, x_14, x_15, x_61); -x_67 = lean_ctor_get(x_66, 0); -lean_inc(x_67); -x_68 = lean_unbox(x_67); -lean_dec(x_67); -if (x_68 == 0) -{ -lean_object* x_69; lean_object* x_70; lean_object* x_71; -lean_free_object(x_58); -lean_dec(x_60); -lean_free_object(x_41); -lean_free_object(x_28); -x_69 = lean_ctor_get(x_66, 1); -lean_inc(x_69); -lean_dec(x_66); -x_70 = lean_box(0); -x_71 = l_Lean_Elab_Command_elabAxiom___lambda__3(x_48, x_2, x_8, x_17, x_70, x_10, x_11, x_12, x_13, x_14, x_15, x_69); -return x_71; -} -else -{ -uint8_t x_72; -x_72 = !lean_is_exclusive(x_66); -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_66, 1); -x_74 = lean_ctor_get(x_66, 0); -lean_dec(x_74); -lean_inc(x_2); -x_75 = l_Lean_MessageData_ofName(x_2); -x_76 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__9; -lean_ctor_set_tag(x_66, 7); -lean_ctor_set(x_66, 1, x_75); -lean_ctor_set(x_66, 0, x_76); -x_77 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__11; -lean_ctor_set_tag(x_58, 7); -lean_ctor_set(x_58, 1, x_77); -lean_ctor_set(x_58, 0, x_66); -x_78 = l_Lean_MessageData_ofExpr(x_60); -lean_ctor_set_tag(x_41, 7); -lean_ctor_set(x_41, 1, x_78); -lean_ctor_set(x_41, 0, x_58); -lean_ctor_set_tag(x_28, 7); -lean_ctor_set(x_28, 1, x_76); -lean_ctor_set(x_28, 0, x_41); -x_79 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_65, x_28, x_10, x_11, x_12, x_13, x_14, x_15, x_73); -x_80 = lean_ctor_get(x_79, 0); -lean_inc(x_80); -x_81 = lean_ctor_get(x_79, 1); -lean_inc(x_81); -lean_dec(x_79); -x_82 = l_Lean_Elab_Command_elabAxiom___lambda__3(x_48, x_2, x_8, x_17, x_80, x_10, x_11, x_12, x_13, x_14, x_15, x_81); -lean_dec(x_80); -return x_82; -} -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; -x_83 = lean_ctor_get(x_66, 1); -lean_inc(x_83); -lean_dec(x_66); -lean_inc(x_2); -x_84 = l_Lean_MessageData_ofName(x_2); -x_85 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__9; -x_86 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_86, 0, x_85); -lean_ctor_set(x_86, 1, x_84); -x_87 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__11; -lean_ctor_set_tag(x_58, 7); -lean_ctor_set(x_58, 1, x_87); -lean_ctor_set(x_58, 0, x_86); -x_88 = l_Lean_MessageData_ofExpr(x_60); -lean_ctor_set_tag(x_41, 7); -lean_ctor_set(x_41, 1, x_88); -lean_ctor_set(x_41, 0, x_58); -lean_ctor_set_tag(x_28, 7); -lean_ctor_set(x_28, 1, x_85); -lean_ctor_set(x_28, 0, x_41); -x_89 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_65, x_28, x_10, x_11, x_12, x_13, x_14, x_15, x_83); -x_90 = lean_ctor_get(x_89, 0); -lean_inc(x_90); -x_91 = lean_ctor_get(x_89, 1); -lean_inc(x_91); -lean_dec(x_89); -x_92 = l_Lean_Elab_Command_elabAxiom___lambda__3(x_48, x_2, x_8, x_17, x_90, x_10, x_11, x_12, x_13, x_14, x_15, x_91); -lean_dec(x_90); -return x_92; -} -} -} -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; uint8_t x_101; -x_93 = lean_ctor_get(x_58, 0); -x_94 = lean_ctor_get(x_58, 1); -lean_inc(x_94); -lean_inc(x_93); -lean_dec(x_58); -lean_inc(x_93); -lean_inc(x_2); -x_95 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_95, 0, x_2); -lean_ctor_set(x_95, 1, x_57); -lean_ctor_set(x_95, 2, x_93); -x_96 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 3); -lean_dec(x_1); -x_97 = lean_alloc_ctor(0, 1, 1); -lean_ctor_set(x_97, 0, x_95); -lean_ctor_set_uint8(x_97, sizeof(void*)*1, x_96); -lean_ctor_set_tag(x_48, 0); -lean_ctor_set(x_48, 0, x_97); -x_98 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__7; -x_99 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_98, x_10, x_11, x_12, x_13, x_14, x_15, x_94); -x_100 = lean_ctor_get(x_99, 0); -lean_inc(x_100); -x_101 = lean_unbox(x_100); -lean_dec(x_100); -if (x_101 == 0) -{ -lean_object* x_102; lean_object* x_103; lean_object* x_104; -lean_dec(x_93); -lean_free_object(x_41); -lean_free_object(x_28); -x_102 = lean_ctor_get(x_99, 1); -lean_inc(x_102); -lean_dec(x_99); -x_103 = lean_box(0); -x_104 = l_Lean_Elab_Command_elabAxiom___lambda__3(x_48, x_2, x_8, x_17, x_103, x_10, x_11, x_12, x_13, x_14, x_15, x_102); -return x_104; -} -else -{ -lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; -x_105 = lean_ctor_get(x_99, 1); -lean_inc(x_105); -if (lean_is_exclusive(x_99)) { - lean_ctor_release(x_99, 0); - lean_ctor_release(x_99, 1); - x_106 = x_99; -} else { - lean_dec_ref(x_99); - x_106 = lean_box(0); -} -lean_inc(x_2); -x_107 = l_Lean_MessageData_ofName(x_2); -x_108 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__9; -if (lean_is_scalar(x_106)) { - x_109 = lean_alloc_ctor(7, 2, 0); -} else { - x_109 = x_106; - lean_ctor_set_tag(x_109, 7); -} -lean_ctor_set(x_109, 0, x_108); -lean_ctor_set(x_109, 1, x_107); -x_110 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__11; -x_111 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_111, 0, x_109); -lean_ctor_set(x_111, 1, x_110); -x_112 = l_Lean_MessageData_ofExpr(x_93); -lean_ctor_set_tag(x_41, 7); -lean_ctor_set(x_41, 1, x_112); -lean_ctor_set(x_41, 0, x_111); -lean_ctor_set_tag(x_28, 7); -lean_ctor_set(x_28, 1, x_108); -lean_ctor_set(x_28, 0, x_41); -x_113 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_98, x_28, x_10, x_11, x_12, x_13, x_14, x_15, x_105); -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 = l_Lean_Elab_Command_elabAxiom___lambda__3(x_48, x_2, x_8, x_17, x_114, x_10, x_11, x_12, x_13, x_14, x_15, x_115); -lean_dec(x_114); -return x_116; -} -} -} -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; uint8_t x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; uint8_t x_129; -x_117 = lean_ctor_get(x_48, 0); -lean_inc(x_117); -lean_dec(x_48); -x_118 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_43, x_10, x_11, x_12, x_13, x_14, x_15, x_44); -x_119 = lean_ctor_get(x_118, 0); -lean_inc(x_119); -x_120 = lean_ctor_get(x_118, 1); -lean_inc(x_120); -if (lean_is_exclusive(x_118)) { - lean_ctor_release(x_118, 0); - lean_ctor_release(x_118, 1); - x_121 = x_118; -} else { - lean_dec_ref(x_118); - x_121 = lean_box(0); -} -lean_inc(x_119); -lean_inc(x_2); -x_122 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_122, 0, x_2); -lean_ctor_set(x_122, 1, x_117); -lean_ctor_set(x_122, 2, x_119); -x_123 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 3); -lean_dec(x_1); -x_124 = lean_alloc_ctor(0, 1, 1); -lean_ctor_set(x_124, 0, x_122); -lean_ctor_set_uint8(x_124, sizeof(void*)*1, x_123); -x_125 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_125, 0, x_124); -x_126 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__7; -x_127 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_126, x_10, x_11, x_12, x_13, x_14, x_15, x_120); -x_128 = lean_ctor_get(x_127, 0); -lean_inc(x_128); -x_129 = lean_unbox(x_128); -lean_dec(x_128); -if (x_129 == 0) -{ -lean_object* x_130; lean_object* x_131; lean_object* x_132; -lean_dec(x_121); -lean_dec(x_119); -lean_free_object(x_41); -lean_free_object(x_28); -x_130 = lean_ctor_get(x_127, 1); -lean_inc(x_130); -lean_dec(x_127); -x_131 = lean_box(0); -x_132 = l_Lean_Elab_Command_elabAxiom___lambda__3(x_125, x_2, x_8, x_17, x_131, x_10, x_11, x_12, x_13, x_14, x_15, x_130); -return x_132; -} -else -{ -lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; -x_133 = lean_ctor_get(x_127, 1); -lean_inc(x_133); -if (lean_is_exclusive(x_127)) { - lean_ctor_release(x_127, 0); - lean_ctor_release(x_127, 1); - x_134 = x_127; -} else { - lean_dec_ref(x_127); - x_134 = lean_box(0); -} -lean_inc(x_2); -x_135 = l_Lean_MessageData_ofName(x_2); -x_136 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__9; -if (lean_is_scalar(x_134)) { - x_137 = lean_alloc_ctor(7, 2, 0); -} else { - x_137 = x_134; - lean_ctor_set_tag(x_137, 7); -} -lean_ctor_set(x_137, 0, x_136); -lean_ctor_set(x_137, 1, x_135); -x_138 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__11; -if (lean_is_scalar(x_121)) { - x_139 = lean_alloc_ctor(7, 2, 0); -} else { - x_139 = x_121; - lean_ctor_set_tag(x_139, 7); -} -lean_ctor_set(x_139, 0, x_137); -lean_ctor_set(x_139, 1, x_138); -x_140 = l_Lean_MessageData_ofExpr(x_119); -lean_ctor_set_tag(x_41, 7); -lean_ctor_set(x_41, 1, x_140); -lean_ctor_set(x_41, 0, x_139); -lean_ctor_set_tag(x_28, 7); -lean_ctor_set(x_28, 1, x_136); -lean_ctor_set(x_28, 0, x_41); -x_141 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_126, x_28, x_10, x_11, x_12, x_13, x_14, x_15, x_133); -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 = l_Lean_Elab_Command_elabAxiom___lambda__3(x_125, x_2, x_8, x_17, x_142, x_10, x_11, x_12, x_13, x_14, x_15, x_143); -lean_dec(x_142); -return x_144; -} -} -} -} -else -{ -lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; -x_145 = lean_ctor_get(x_41, 0); -x_146 = lean_ctor_get(x_41, 1); -lean_inc(x_146); -lean_inc(x_145); -lean_dec(x_41); -x_147 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__5; -lean_inc(x_145); -x_148 = l_Lean_CollectLevelParams_main(x_145, x_147); -x_149 = lean_ctor_get(x_148, 2); -lean_inc(x_149); -lean_dec(x_148); -x_150 = l_Lean_Elab_sortDeclLevelParams(x_5, x_6, x_149); -if (lean_obj_tag(x_150) == 0) -{ -lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; -lean_dec(x_145); -lean_free_object(x_28); -lean_dec(x_17); -lean_dec(x_8); -lean_dec(x_2); -lean_dec(x_1); -x_151 = lean_ctor_get(x_150, 0); -lean_inc(x_151); -if (lean_is_exclusive(x_150)) { - lean_ctor_release(x_150, 0); - x_152 = x_150; -} else { - lean_dec_ref(x_150); - x_152 = lean_box(0); -} -if (lean_is_scalar(x_152)) { - x_153 = lean_alloc_ctor(3, 1, 0); -} else { - x_153 = x_152; - lean_ctor_set_tag(x_153, 3); -} -lean_ctor_set(x_153, 0, x_151); -x_154 = l_Lean_MessageData_ofFormat(x_153); -x_155 = l_Lean_throwErrorAt___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__12(x_7, x_154, x_10, x_11, x_12, x_13, x_14, x_15, x_146); -lean_dec(x_15); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -return x_155; -} -else -{ -lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; uint8_t x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; uint8_t x_169; -x_156 = lean_ctor_get(x_150, 0); -lean_inc(x_156); -if (lean_is_exclusive(x_150)) { - lean_ctor_release(x_150, 0); - x_157 = x_150; -} else { - lean_dec_ref(x_150); - x_157 = lean_box(0); -} -x_158 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_145, x_10, x_11, x_12, x_13, x_14, x_15, x_146); -x_159 = lean_ctor_get(x_158, 0); -lean_inc(x_159); -x_160 = lean_ctor_get(x_158, 1); -lean_inc(x_160); -if (lean_is_exclusive(x_158)) { - lean_ctor_release(x_158, 0); - lean_ctor_release(x_158, 1); - x_161 = x_158; -} else { - lean_dec_ref(x_158); - x_161 = lean_box(0); -} -lean_inc(x_159); -lean_inc(x_2); -x_162 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_162, 0, x_2); -lean_ctor_set(x_162, 1, x_156); -lean_ctor_set(x_162, 2, x_159); -x_163 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 3); -lean_dec(x_1); -x_164 = lean_alloc_ctor(0, 1, 1); -lean_ctor_set(x_164, 0, x_162); -lean_ctor_set_uint8(x_164, sizeof(void*)*1, x_163); -if (lean_is_scalar(x_157)) { - x_165 = lean_alloc_ctor(0, 1, 0); -} else { - x_165 = x_157; - lean_ctor_set_tag(x_165, 0); -} -lean_ctor_set(x_165, 0, x_164); -x_166 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__7; -x_167 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_166, x_10, x_11, x_12, x_13, x_14, x_15, x_160); -x_168 = lean_ctor_get(x_167, 0); -lean_inc(x_168); -x_169 = lean_unbox(x_168); -lean_dec(x_168); -if (x_169 == 0) -{ -lean_object* x_170; lean_object* x_171; lean_object* x_172; -lean_dec(x_161); -lean_dec(x_159); -lean_free_object(x_28); -x_170 = lean_ctor_get(x_167, 1); -lean_inc(x_170); -lean_dec(x_167); -x_171 = lean_box(0); -x_172 = l_Lean_Elab_Command_elabAxiom___lambda__3(x_165, x_2, x_8, x_17, x_171, x_10, x_11, x_12, x_13, x_14, x_15, x_170); -return x_172; -} -else -{ -lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; -x_173 = lean_ctor_get(x_167, 1); -lean_inc(x_173); -if (lean_is_exclusive(x_167)) { - lean_ctor_release(x_167, 0); - lean_ctor_release(x_167, 1); - x_174 = x_167; -} else { - lean_dec_ref(x_167); - x_174 = lean_box(0); -} -lean_inc(x_2); -x_175 = l_Lean_MessageData_ofName(x_2); -x_176 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__9; -if (lean_is_scalar(x_174)) { - x_177 = lean_alloc_ctor(7, 2, 0); -} else { - x_177 = x_174; - lean_ctor_set_tag(x_177, 7); -} -lean_ctor_set(x_177, 0, x_176); -lean_ctor_set(x_177, 1, x_175); -x_178 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__11; -if (lean_is_scalar(x_161)) { - x_179 = lean_alloc_ctor(7, 2, 0); -} else { - x_179 = x_161; - lean_ctor_set_tag(x_179, 7); -} -lean_ctor_set(x_179, 0, x_177); -lean_ctor_set(x_179, 1, x_178); -x_180 = l_Lean_MessageData_ofExpr(x_159); -x_181 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_181, 0, x_179); -lean_ctor_set(x_181, 1, x_180); -lean_ctor_set_tag(x_28, 7); -lean_ctor_set(x_28, 1, x_176); -lean_ctor_set(x_28, 0, x_181); -x_182 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_166, x_28, x_10, x_11, x_12, x_13, x_14, x_15, x_173); -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_Elab_Command_elabAxiom___lambda__3(x_165, x_2, x_8, x_17, x_183, x_10, x_11, x_12, x_13, x_14, x_15, x_184); -lean_dec(x_183); -return x_185; -} -} -} -} -else -{ -uint8_t x_186; -lean_free_object(x_28); -lean_dec(x_17); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_8); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_2); -lean_dec(x_1); -x_186 = !lean_is_exclusive(x_37); -if (x_186 == 0) -{ -return x_37; -} -else -{ -lean_object* x_187; lean_object* x_188; lean_object* x_189; -x_187 = lean_ctor_get(x_37, 0); -x_188 = lean_ctor_get(x_37, 1); -lean_inc(x_188); -lean_inc(x_187); -lean_dec(x_37); -x_189 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_189, 0, x_187); -lean_ctor_set(x_189, 1, x_188); -return x_189; -} -} -} -else -{ -uint8_t x_190; -lean_free_object(x_28); -lean_dec(x_17); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_8); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -x_190 = !lean_is_exclusive(x_34); -if (x_190 == 0) -{ -return x_34; -} -else -{ -lean_object* x_191; lean_object* x_192; lean_object* x_193; -x_191 = lean_ctor_get(x_34, 0); -x_192 = lean_ctor_get(x_34, 1); -lean_inc(x_192); -lean_inc(x_191); -lean_dec(x_34); -x_193 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_193, 0, x_191); -lean_ctor_set(x_193, 1, x_192); -return x_193; -} -} -} -else -{ -lean_object* x_194; lean_object* x_195; uint8_t x_196; uint8_t x_197; lean_object* x_198; -x_194 = lean_ctor_get(x_28, 0); -x_195 = lean_ctor_get(x_28, 1); -lean_inc(x_195); -lean_inc(x_194); -lean_dec(x_28); -x_196 = 1; -x_197 = 1; -x_198 = l_Lean_Meta_mkForallFVars(x_9, x_194, x_25, x_196, x_197, x_12, x_13, x_14, x_15, x_195); -if (lean_obj_tag(x_198) == 0) -{ -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_198, 1); -lean_inc(x_200); -lean_dec(x_198); -x_201 = l_Lean_Meta_mkForallFVars(x_4, x_199, x_196, x_196, x_197, x_12, x_13, x_14, x_15, x_200); -if (lean_obj_tag(x_201) == 0) -{ -lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; -x_202 = lean_ctor_get(x_201, 0); -lean_inc(x_202); -x_203 = lean_ctor_get(x_201, 1); -lean_inc(x_203); -lean_dec(x_201); -x_204 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_ensureValidNamespace___closed__2; -x_205 = l_Lean_Elab_Term_levelMVarToParam(x_202, x_204, x_10, x_11, x_12, x_13, x_14, x_15, x_203); -x_206 = lean_ctor_get(x_205, 0); -lean_inc(x_206); -x_207 = lean_ctor_get(x_205, 1); -lean_inc(x_207); -if (lean_is_exclusive(x_205)) { - lean_ctor_release(x_205, 0); - lean_ctor_release(x_205, 1); - x_208 = x_205; -} else { - lean_dec_ref(x_205); - x_208 = lean_box(0); -} -x_209 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__5; -lean_inc(x_206); -x_210 = l_Lean_CollectLevelParams_main(x_206, x_209); -x_211 = lean_ctor_get(x_210, 2); -lean_inc(x_211); -lean_dec(x_210); -x_212 = l_Lean_Elab_sortDeclLevelParams(x_5, x_6, x_211); -if (lean_obj_tag(x_212) == 0) -{ -lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; -lean_dec(x_208); -lean_dec(x_206); -lean_dec(x_17); -lean_dec(x_8); -lean_dec(x_2); -lean_dec(x_1); -x_213 = lean_ctor_get(x_212, 0); -lean_inc(x_213); -if (lean_is_exclusive(x_212)) { - lean_ctor_release(x_212, 0); - x_214 = x_212; -} else { - lean_dec_ref(x_212); - x_214 = lean_box(0); -} -if (lean_is_scalar(x_214)) { - x_215 = lean_alloc_ctor(3, 1, 0); -} else { - x_215 = x_214; - lean_ctor_set_tag(x_215, 3); -} -lean_ctor_set(x_215, 0, x_213); -x_216 = l_Lean_MessageData_ofFormat(x_215); -x_217 = l_Lean_throwErrorAt___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__12(x_7, x_216, x_10, x_11, x_12, x_13, x_14, x_15, x_207); -lean_dec(x_15); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -return x_217; -} -else -{ -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; uint8_t x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; uint8_t x_231; -x_218 = lean_ctor_get(x_212, 0); -lean_inc(x_218); -if (lean_is_exclusive(x_212)) { - lean_ctor_release(x_212, 0); - x_219 = x_212; -} else { - lean_dec_ref(x_212); - x_219 = lean_box(0); -} -x_220 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_206, x_10, x_11, x_12, x_13, x_14, x_15, x_207); -x_221 = lean_ctor_get(x_220, 0); -lean_inc(x_221); -x_222 = lean_ctor_get(x_220, 1); -lean_inc(x_222); -if (lean_is_exclusive(x_220)) { - lean_ctor_release(x_220, 0); - lean_ctor_release(x_220, 1); - x_223 = x_220; -} else { - lean_dec_ref(x_220); - x_223 = lean_box(0); -} -lean_inc(x_221); -lean_inc(x_2); -x_224 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_224, 0, x_2); -lean_ctor_set(x_224, 1, x_218); -lean_ctor_set(x_224, 2, x_221); -x_225 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 3); -lean_dec(x_1); -x_226 = lean_alloc_ctor(0, 1, 1); -lean_ctor_set(x_226, 0, x_224); -lean_ctor_set_uint8(x_226, sizeof(void*)*1, x_225); -if (lean_is_scalar(x_219)) { - x_227 = lean_alloc_ctor(0, 1, 0); -} else { - x_227 = x_219; - lean_ctor_set_tag(x_227, 0); -} -lean_ctor_set(x_227, 0, x_226); -x_228 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__7; -x_229 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_228, x_10, x_11, x_12, x_13, x_14, x_15, x_222); -x_230 = lean_ctor_get(x_229, 0); -lean_inc(x_230); -x_231 = lean_unbox(x_230); -lean_dec(x_230); -if (x_231 == 0) -{ -lean_object* x_232; lean_object* x_233; lean_object* x_234; -lean_dec(x_223); -lean_dec(x_221); -lean_dec(x_208); -x_232 = lean_ctor_get(x_229, 1); -lean_inc(x_232); -lean_dec(x_229); -x_233 = lean_box(0); -x_234 = l_Lean_Elab_Command_elabAxiom___lambda__3(x_227, x_2, x_8, x_17, x_233, x_10, x_11, x_12, x_13, x_14, x_15, x_232); -return x_234; -} -else -{ -lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; -x_235 = lean_ctor_get(x_229, 1); -lean_inc(x_235); -if (lean_is_exclusive(x_229)) { - lean_ctor_release(x_229, 0); - lean_ctor_release(x_229, 1); - x_236 = x_229; -} else { - lean_dec_ref(x_229); - x_236 = lean_box(0); -} -lean_inc(x_2); -x_237 = l_Lean_MessageData_ofName(x_2); -x_238 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__9; -if (lean_is_scalar(x_236)) { - x_239 = lean_alloc_ctor(7, 2, 0); -} else { - x_239 = x_236; - lean_ctor_set_tag(x_239, 7); -} -lean_ctor_set(x_239, 0, x_238); -lean_ctor_set(x_239, 1, x_237); -x_240 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__11; -if (lean_is_scalar(x_223)) { - x_241 = lean_alloc_ctor(7, 2, 0); -} else { - x_241 = x_223; - lean_ctor_set_tag(x_241, 7); -} -lean_ctor_set(x_241, 0, x_239); -lean_ctor_set(x_241, 1, x_240); -x_242 = l_Lean_MessageData_ofExpr(x_221); -if (lean_is_scalar(x_208)) { - x_243 = lean_alloc_ctor(7, 2, 0); -} else { - x_243 = x_208; - lean_ctor_set_tag(x_243, 7); -} -lean_ctor_set(x_243, 0, x_241); -lean_ctor_set(x_243, 1, x_242); -x_244 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_244, 0, x_243); -lean_ctor_set(x_244, 1, x_238); -x_245 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_228, x_244, x_10, x_11, x_12, x_13, x_14, x_15, x_235); -x_246 = lean_ctor_get(x_245, 0); -lean_inc(x_246); -x_247 = lean_ctor_get(x_245, 1); -lean_inc(x_247); -lean_dec(x_245); -x_248 = l_Lean_Elab_Command_elabAxiom___lambda__3(x_227, x_2, x_8, x_17, x_246, x_10, x_11, x_12, x_13, x_14, x_15, x_247); -lean_dec(x_246); -return x_248; -} -} -} -else -{ -lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; -lean_dec(x_17); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_8); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_2); -lean_dec(x_1); -x_249 = lean_ctor_get(x_201, 0); -lean_inc(x_249); -x_250 = lean_ctor_get(x_201, 1); -lean_inc(x_250); -if (lean_is_exclusive(x_201)) { - lean_ctor_release(x_201, 0); - lean_ctor_release(x_201, 1); - x_251 = x_201; -} else { - lean_dec_ref(x_201); - x_251 = lean_box(0); -} -if (lean_is_scalar(x_251)) { - x_252 = lean_alloc_ctor(1, 2, 0); -} else { - x_252 = x_251; -} -lean_ctor_set(x_252, 0, x_249); -lean_ctor_set(x_252, 1, x_250); -return x_252; -} -} -else -{ -lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; -lean_dec(x_17); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_8); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -x_253 = lean_ctor_get(x_198, 0); -lean_inc(x_253); -x_254 = lean_ctor_get(x_198, 1); -lean_inc(x_254); -if (lean_is_exclusive(x_198)) { - lean_ctor_release(x_198, 0); - lean_ctor_release(x_198, 1); - x_255 = x_198; -} else { - lean_dec_ref(x_198); - x_255 = lean_box(0); -} -if (lean_is_scalar(x_255)) { - x_256 = lean_alloc_ctor(1, 2, 0); -} else { - x_256 = x_255; -} -lean_ctor_set(x_256, 0, x_253); -lean_ctor_set(x_256, 1, x_254); -return x_256; -} -} -} -else -{ -uint8_t x_257; -lean_dec(x_22); -lean_dec(x_17); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -x_257 = !lean_is_exclusive(x_26); -if (x_257 == 0) -{ -return x_26; -} -else -{ -lean_object* x_258; lean_object* x_259; lean_object* x_260; -x_258 = lean_ctor_get(x_26, 0); -x_259 = lean_ctor_get(x_26, 1); -lean_inc(x_259); -lean_inc(x_258); -lean_dec(x_26); -x_260 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_260, 0, x_258); -lean_ctor_set(x_260, 1, x_259); -return x_260; -} -} -} -else -{ -uint8_t x_261; -lean_dec(x_17); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -x_261 = !lean_is_exclusive(x_21); -if (x_261 == 0) -{ -return x_21; -} -else -{ -lean_object* x_262; lean_object* x_263; lean_object* x_264; -x_262 = lean_ctor_get(x_21, 0); -x_263 = lean_ctor_get(x_21, 1); -lean_inc(x_263); -lean_inc(x_262); -lean_dec(x_21); -x_264 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_264, 0, x_262); -lean_ctor_set(x_264, 1, x_263); -return x_264; -} -} -} -else -{ -uint8_t x_265; -lean_dec(x_17); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_265 = !lean_is_exclusive(x_19); -if (x_265 == 0) -{ -return x_19; -} -else -{ -lean_object* x_266; lean_object* x_267; lean_object* x_268; -x_266 = lean_ctor_get(x_19, 0); -x_267 = lean_ctor_get(x_19, 1); -lean_inc(x_267); -lean_inc(x_266); -lean_dec(x_19); -x_268 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_268, 0, x_266); -lean_ctor_set(x_268, 1, x_267); -return x_268; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___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) { -_start: -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_17 = l_Lean_Syntax_getArgs(x_1); -lean_inc(x_6); -lean_inc(x_3); -x_18 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabAxiom___lambda__4___boxed), 16, 8); -lean_closure_set(x_18, 0, x_2); -lean_closure_set(x_18, 1, x_3); -lean_closure_set(x_18, 2, x_4); -lean_closure_set(x_18, 3, x_9); -lean_closure_set(x_18, 4, x_5); -lean_closure_set(x_18, 5, x_6); -lean_closure_set(x_18, 6, x_7); -lean_closure_set(x_18, 7, x_8); -x_19 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabBinders___rarg), 9, 2); -lean_closure_set(x_19, 0, x_17); -lean_closure_set(x_19, 1, x_18); -x_20 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withLevelNames___rarg), 9, 2); -lean_closure_set(x_20, 0, x_6); -lean_closure_set(x_20, 1, x_19); -x_21 = l_Lean_Elab_Term_withDeclName___rarg(x_3, x_20, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -return x_21; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom(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; -x_6 = lean_unsigned_to_nat(1u); -x_7 = l_Lean_Syntax_getArg(x_2, x_6); -x_8 = lean_unsigned_to_nat(2u); -x_9 = l_Lean_Syntax_getArg(x_2, x_8); -x_10 = l_Lean_Elab_expandDeclSig(x_9); -lean_dec(x_9); -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -x_12 = lean_ctor_get(x_10, 1); -lean_inc(x_12); -lean_dec(x_10); -x_13 = l_Lean_Elab_Command_getLevelNames___rarg(x_4, x_5); -x_14 = lean_ctor_get(x_13, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_13, 1); -lean_inc(x_15); -lean_dec(x_13); -lean_inc(x_3); -lean_inc(x_1); -x_16 = l_Lean_Elab_Command_expandDeclId(x_7, x_1, x_3, x_4, x_15); -if (lean_obj_tag(x_16) == 0) -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_16, 1); -lean_inc(x_18); -lean_dec(x_16); -x_19 = lean_ctor_get(x_17, 1); -lean_inc(x_19); -x_20 = lean_ctor_get(x_17, 2); -lean_inc(x_20); -lean_dec(x_17); -lean_inc(x_3); -lean_inc(x_2); -lean_inc(x_19); -x_21 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1(x_19, x_2, x_3, x_4, x_18); -x_22 = lean_ctor_get(x_21, 1); -lean_inc(x_22); -lean_dec(x_21); -x_23 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabAxiom___lambda__5___boxed), 16, 8); -lean_closure_set(x_23, 0, x_11); -lean_closure_set(x_23, 1, x_1); -lean_closure_set(x_23, 2, x_19); -lean_closure_set(x_23, 3, x_12); -lean_closure_set(x_23, 4, x_14); -lean_closure_set(x_23, 5, x_20); -lean_closure_set(x_23, 6, x_2); -lean_closure_set(x_23, 7, x_7); -x_24 = l_Lean_Elab_Command_runTermElabM___rarg(x_23, x_3, x_4, x_22); -lean_dec(x_3); -return x_24; -} -else -{ -uint8_t x_25; -lean_dec(x_14); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_25 = !lean_is_exclusive(x_16); -if (x_25 == 0) -{ -return x_16; -} -else -{ -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_16, 0); -x_27 = lean_ctor_get(x_16, 1); -lean_inc(x_27); -lean_inc(x_26); -lean_dec(x_16); -x_28 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_28, 0, x_26); -lean_ctor_set(x_28, 1, x_27); -return x_28; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Command_elabAxiom___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -lean_object* x_5; -x_5 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Command_elabAxiom___spec__2(x_1, x_2, x_3, x_4); -lean_dec(x_3); -lean_dec(x_1); -return x_5; -} -} -LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; -x_6 = l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__3(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_4); -lean_dec(x_3); -return x_6; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; -x_6 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_4); -return x_6; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; -x_11 = l_Lean_Elab_Command_elabAxiom___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_3); -return x_11; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -lean_object* x_13; -x_13 = l_Lean_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, x_11, x_12); -lean_dec(x_5); -return x_13; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: -{ -lean_object* x_17; -x_17 = l_Lean_Elab_Command_elabAxiom___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_7); -return x_17; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: -{ -lean_object* x_17; -x_17 = l_Lean_Elab_Command_elabAxiom___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); -lean_dec(x_1); -return x_17; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; -x_6 = l_Lean_Elab_Command_elabAxiom(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_4); -return x_6; -} -} -static lean_object* _init_l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__1___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("invalid use of attributes in constructor declaration", 52, 52); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__1___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__1___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -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* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; -x_6 = lean_ctor_get(x_1, 1); -x_7 = lean_array_get_size(x_6); -x_8 = lean_unsigned_to_nat(0u); -x_9 = lean_nat_dec_eq(x_7, x_8); -lean_dec(x_7); -if (x_9 == 0) -{ -lean_object* x_10; lean_object* x_11; -x_10 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__1___closed__2; -x_11 = l_Lean_throwError___at___private_Lean_Elab_Command_0__Lean_Elab_Command_elabCommandUsing___spec__1(x_10, x_3, x_4, x_5); -return x_11; -} -else -{ -lean_object* x_12; lean_object* x_13; -lean_dec(x_3); -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_5); -return x_13; -} -} -} -static lean_object* _init_l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__2___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("invalid use of 'unsafe' in constructor declaration", 50, 50); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__2___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__2___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -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* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -uint8_t x_6; -x_6 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 3); -if (x_6 == 0) -{ -lean_object* x_7; lean_object* x_8; -x_7 = lean_box(0); -x_8 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__1(x_1, x_7, x_3, x_4, x_5); -return x_8; -} -else -{ -lean_object* x_9; lean_object* x_10; uint8_t x_11; -x_9 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__2___closed__2; -x_10 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_9, x_3, x_4, x_5); -x_11 = !lean_is_exclusive(x_10); -if (x_11 == 0) -{ -return x_10; -} -else -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_12 = lean_ctor_get(x_10, 0); -x_13 = lean_ctor_get(x_10, 1); -lean_inc(x_13); -lean_inc(x_12); -lean_dec(x_10); -x_14 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_14, 0, x_12); -lean_ctor_set(x_14, 1, x_13); -return x_14; -} -} -} -} -static lean_object* _init_l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__3___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("invalid use of 'partial' in constructor declaration", 51, 51); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__3___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__3___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -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* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -uint8_t x_6; -x_6 = l_Lean_Elab_Modifiers_isPartial(x_1); -if (x_6 == 0) -{ -lean_object* x_7; lean_object* x_8; -x_7 = lean_box(0); -x_8 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__2(x_1, x_7, x_3, x_4, x_5); -return x_8; -} -else -{ -lean_object* x_9; lean_object* x_10; uint8_t x_11; -x_9 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__3___closed__2; -x_10 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_9, x_3, x_4, x_5); -x_11 = !lean_is_exclusive(x_10); -if (x_11 == 0) -{ -return x_10; -} -else -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_12 = lean_ctor_get(x_10, 0); -x_13 = lean_ctor_get(x_10, 1); -lean_inc(x_13); -lean_inc(x_12); -lean_dec(x_10); -x_14 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_14, 0, x_12); -lean_ctor_set(x_14, 1, x_13); -return x_14; -} -} -} -} -static lean_object* _init_l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("invalid use of 'noncomputable' in constructor declaration", 57, 57); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -uint8_t x_5; -x_5 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 1); -if (x_5 == 0) -{ -lean_object* x_6; lean_object* x_7; -x_6 = lean_box(0); -x_7 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__3(x_1, x_6, x_2, x_3, x_4); -return x_7; -} -else -{ -lean_object* x_8; lean_object* x_9; uint8_t x_10; -x_8 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___closed__2; -x_9 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_8, x_2, x_3, x_4); -x_10 = !lean_is_exclusive(x_9); -if (x_10 == 0) -{ -return x_9; -} -else -{ -lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_11 = lean_ctor_get(x_9, 0); -x_12 = lean_ctor_get(x_9, 1); -lean_inc(x_12); -lean_inc(x_11); -lean_dec(x_9); -x_13 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_13, 0, x_11); -lean_ctor_set(x_13, 1, x_12); -return x_13; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; -lean_inc(x_4); -x_7 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Command_elabAxiom___spec__2(x_2, x_4, x_5, x_6); -x_8 = lean_ctor_get(x_7, 0); -lean_inc(x_8); -x_9 = lean_ctor_get(x_7, 1); -lean_inc(x_9); -lean_dec(x_7); -lean_inc(x_4); -x_10 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Command_elabAxiom___spec__2(x_3, x_4, x_5, x_9); -x_11 = !lean_is_exclusive(x_10); -if (x_11 == 0) -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_12 = lean_ctor_get(x_10, 0); -x_13 = lean_ctor_get(x_10, 1); -lean_ctor_set(x_10, 1, x_12); -lean_ctor_set(x_10, 0, x_8); -x_14 = l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__3(x_1, x_10, x_4, x_5, x_13); -lean_dec(x_4); -return x_14; -} -else -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_15 = lean_ctor_get(x_10, 0); -x_16 = lean_ctor_get(x_10, 1); -lean_inc(x_16); -lean_inc(x_15); -lean_dec(x_10); -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_8); -lean_ctor_set(x_17, 1, x_15); -x_18 = l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__3(x_1, x_17, x_4, x_5, x_16); -lean_dec(x_4); -return x_18; -} -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___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) { -_start: -{ -lean_object* x_8; -lean_inc(x_5); -x_8 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1(x_1, x_5, x_6, x_7); -if (lean_obj_tag(x_8) == 0) -{ -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; lean_object* x_15; lean_object* x_16; 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; -x_9 = lean_ctor_get(x_8, 1); -lean_inc(x_9); -lean_dec(x_8); -x_10 = lean_unsigned_to_nat(3u); -x_11 = l_Lean_Syntax_getIdAt(x_2, x_10); -x_12 = l_Lean_Name_append(x_3, x_11); -x_13 = l_Lean_Syntax_getArg(x_2, x_10); -x_14 = lean_ctor_get_uint8(x_1, sizeof(void*)*2); -x_15 = l_Lean_Elab_Command_getRef(x_5, x_6, x_9); -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_replaceRef(x_13, x_16); -lean_dec(x_16); -x_19 = lean_ctor_get(x_5, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_5, 1); -lean_inc(x_20); -x_21 = lean_ctor_get(x_5, 2); -lean_inc(x_21); -x_22 = lean_ctor_get(x_5, 3); -lean_inc(x_22); -x_23 = lean_ctor_get(x_5, 4); -lean_inc(x_23); -x_24 = lean_ctor_get(x_5, 5); -lean_inc(x_24); -x_25 = lean_ctor_get(x_5, 7); -lean_inc(x_25); -x_26 = lean_ctor_get(x_5, 8); -lean_inc(x_26); -x_27 = lean_ctor_get(x_5, 9); -lean_inc(x_27); -x_28 = lean_ctor_get_uint8(x_5, sizeof(void*)*10); -x_29 = lean_alloc_ctor(0, 10, 1); -lean_ctor_set(x_29, 0, x_19); -lean_ctor_set(x_29, 1, x_20); -lean_ctor_set(x_29, 2, x_21); -lean_ctor_set(x_29, 3, x_22); -lean_ctor_set(x_29, 4, x_23); -lean_ctor_set(x_29, 5, x_24); -lean_ctor_set(x_29, 6, x_18); -lean_ctor_set(x_29, 7, x_25); -lean_ctor_set(x_29, 8, x_26); -lean_ctor_set(x_29, 9, x_27); -lean_ctor_set_uint8(x_29, sizeof(void*)*10, x_28); -x_30 = l_Lean_Elab_applyVisibility___at_Lean_Elab_Command_expandDeclId___spec__6(x_14, x_12, x_29, x_6, x_17); -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; lean_object* x_39; -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_unsigned_to_nat(4u); -x_34 = l_Lean_Syntax_getArg(x_2, x_33); -x_35 = l_Lean_Elab_expandOptDeclSig(x_34); -lean_dec(x_34); -x_36 = lean_ctor_get(x_35, 0); -lean_inc(x_36); -x_37 = lean_ctor_get(x_35, 1); -lean_inc(x_37); -lean_dec(x_35); -x_38 = lean_ctor_get(x_1, 0); -lean_inc(x_38); -lean_inc(x_5); -lean_inc(x_31); -x_39 = l_Lean_addDocString_x27___at_Lean_Elab_Command_expandDeclId___spec__13(x_31, x_38, x_5, x_6, x_32); -if (lean_obj_tag(x_39) == 0) -{ -lean_object* x_40; lean_object* x_41; uint8_t x_42; -x_40 = lean_ctor_get(x_39, 1); -lean_inc(x_40); -lean_dec(x_39); -lean_inc(x_31); -x_41 = l_Lean_Elab_addAuxDeclarationRanges___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2(x_31, x_2, x_13, x_5, x_6, x_40); -lean_dec(x_13); -x_42 = !lean_is_exclusive(x_41); -if (x_42 == 0) -{ -lean_object* x_43; lean_object* x_44; -x_43 = lean_ctor_get(x_41, 0); -lean_dec(x_43); -x_44 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_44, 0, x_2); -lean_ctor_set(x_44, 1, x_1); -lean_ctor_set(x_44, 2, x_31); -lean_ctor_set(x_44, 3, x_36); -lean_ctor_set(x_44, 4, x_37); -lean_ctor_set(x_41, 0, x_44); -return x_41; -} -else -{ -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_41, 1); -lean_inc(x_45); -lean_dec(x_41); -x_46 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_46, 0, x_2); -lean_ctor_set(x_46, 1, x_1); -lean_ctor_set(x_46, 2, x_31); -lean_ctor_set(x_46, 3, x_36); -lean_ctor_set(x_46, 4, x_37); -x_47 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_47, 0, x_46); -lean_ctor_set(x_47, 1, x_45); -return x_47; -} -} -else -{ -uint8_t x_48; -lean_dec(x_37); -lean_dec(x_36); -lean_dec(x_31); -lean_dec(x_13); -lean_dec(x_5); -lean_dec(x_2); -lean_dec(x_1); -x_48 = !lean_is_exclusive(x_39); -if (x_48 == 0) -{ -return x_39; -} -else -{ -lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_49 = lean_ctor_get(x_39, 0); -x_50 = lean_ctor_get(x_39, 1); -lean_inc(x_50); -lean_inc(x_49); -lean_dec(x_39); -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_13); -lean_dec(x_5); -lean_dec(x_2); -lean_dec(x_1); -x_52 = !lean_is_exclusive(x_30); -if (x_52 == 0) -{ -return x_30; -} -else -{ -lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_53 = lean_ctor_get(x_30, 0); -x_54 = lean_ctor_get(x_30, 1); -lean_inc(x_54); -lean_inc(x_53); -lean_dec(x_30); -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_56; -lean_dec(x_5); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_56 = !lean_is_exclusive(x_8); -if (x_56 == 0) -{ -return x_8; -} -else -{ -lean_object* x_57; lean_object* x_58; lean_object* x_59; -x_57 = lean_ctor_get(x_8, 0); -x_58 = lean_ctor_get(x_8, 1); -lean_inc(x_58); -lean_inc(x_57); -lean_dec(x_8); -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; -} -} -} -} -static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__2___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("invalid 'protected' constructor in a 'private' inductive datatype", 65, 65); -return x_1; -} -} -static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__2___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__2___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -uint8_t x_9; -x_9 = l_Lean_Elab_Modifiers_isProtected(x_1); -if (x_9 == 0) -{ -lean_object* x_10; lean_object* x_11; -x_10 = lean_box(0); -x_11 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__1(x_1, x_2, x_3, x_10, x_6, x_7, x_8); -return x_11; -} -else -{ -uint8_t x_12; -x_12 = l_Lean_Elab_Modifiers_isPrivate(x_4); -if (x_12 == 0) -{ -lean_object* x_13; lean_object* x_14; -x_13 = lean_box(0); -x_14 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__1(x_1, x_2, x_3, x_13, x_6, x_7, x_8); -return x_14; -} -else -{ -lean_object* x_15; lean_object* x_16; uint8_t x_17; -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_15 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__2___closed__2; -x_16 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_15, x_6, x_7, x_8); -x_17 = !lean_is_exclusive(x_16); -if (x_17 == 0) -{ -return x_16; -} -else -{ -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_16, 0); -x_19 = lean_ctor_get(x_16, 1); -lean_inc(x_19); -lean_inc(x_18); -lean_dec(x_16); -x_20 = lean_alloc_ctor(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_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__3___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("invalid 'private' constructor in a 'private' inductive datatype", 63, 63); -return x_1; -} -} -static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__3___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__3___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -uint8_t x_9; -x_9 = l_Lean_Elab_Modifiers_isPrivate(x_4); -if (x_9 == 0) +x_24 = lean_st_ref_get(x_11, x_23); +x_25 = lean_ctor_get(x_24, 0); +lean_inc(x_25); +x_26 = lean_ctor_get(x_24, 1); +lean_inc(x_26); +lean_dec(x_24); +x_27 = lean_ctor_get(x_25, 0); +lean_inc(x_27); +lean_dec(x_25); +lean_inc(x_2); +x_28 = l_Lean_isExtern(x_27, x_2); +lean_dec(x_27); +if (x_28 == 0) { -lean_object* x_10; lean_object* x_11; -x_10 = lean_box(0); -x_11 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__2(x_4, x_1, x_2, x_3, x_10, x_6, x_7, x_8); -return x_11; +uint8_t x_29; lean_object* x_30; +lean_dec(x_1); +x_29 = 1; +x_30 = l_Lean_Elab_Term_applyAttributesAt(x_2, x_4, x_29, x_6, x_7, x_8, x_9, x_10, x_11, x_26); +return x_30; } else { -uint8_t x_12; -x_12 = l_Lean_Elab_Modifiers_isPrivate(x_3); -if (x_12 == 0) +lean_object* x_31; +lean_inc(x_11); +lean_inc(x_10); +x_31 = l_Lean_compileDecl(x_1, x_10, x_11, x_26); +if (lean_obj_tag(x_31) == 0) { -lean_object* x_13; lean_object* x_14; -x_13 = lean_box(0); -x_14 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__2(x_4, x_1, x_2, x_3, x_13, x_6, x_7, x_8); -return x_14; +lean_object* x_32; uint8_t x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_31, 1); +lean_inc(x_32); +lean_dec(x_31); +x_33 = 1; +x_34 = l_Lean_Elab_Term_applyAttributesAt(x_2, x_4, x_33, x_6, x_7, x_8, x_9, x_10, x_11, x_32); +return x_34; } else { -lean_object* x_15; lean_object* x_16; uint8_t x_17; +uint8_t x_35; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); lean_dec(x_4); lean_dec(x_2); -lean_dec(x_1); -x_15 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__3___closed__2; -x_16 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_15, x_6, x_7, x_8); -x_17 = !lean_is_exclusive(x_16); -if (x_17 == 0) -{ -return x_16; -} -else -{ -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_16, 0); -x_19 = lean_ctor_get(x_16, 1); -lean_inc(x_19); -lean_inc(x_18); -lean_dec(x_16); -x_20 = lean_alloc_ctor(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_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; lean_object* x_9; uint8_t x_10; -x_8 = l_Lean_TSyntax_getDocString(x_1); -x_9 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_9, 0, x_8); -x_10 = !lean_is_exclusive(x_3); -if (x_10 == 0) +x_35 = !lean_is_exclusive(x_31); +if (x_35 == 0) { -lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_11 = lean_ctor_get(x_3, 0); -lean_dec(x_11); -lean_ctor_set(x_3, 0, x_9); -x_12 = lean_box(0); -x_13 = lean_apply_5(x_2, x_3, x_12, x_5, x_6, x_7); -return x_13; +return x_31; } else { -uint8_t x_14; uint8_t x_15; uint8_t x_16; uint8_t x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_14 = lean_ctor_get_uint8(x_3, sizeof(void*)*2); -x_15 = lean_ctor_get_uint8(x_3, sizeof(void*)*2 + 1); -x_16 = lean_ctor_get_uint8(x_3, sizeof(void*)*2 + 2); -x_17 = lean_ctor_get_uint8(x_3, sizeof(void*)*2 + 3); -x_18 = lean_ctor_get(x_3, 1); -lean_inc(x_18); -lean_dec(x_3); -x_19 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_19, 0, x_9); -lean_ctor_set(x_19, 1, x_18); -lean_ctor_set_uint8(x_19, sizeof(void*)*2, x_14); -lean_ctor_set_uint8(x_19, sizeof(void*)*2 + 1, x_15); -lean_ctor_set_uint8(x_19, sizeof(void*)*2 + 2, x_16); -lean_ctor_set_uint8(x_19, sizeof(void*)*2 + 3, x_17); -x_20 = lean_box(0); -x_21 = lean_apply_5(x_2, x_19, x_20, x_5, x_6, x_7); -return x_21; -} -} -} -static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("duplicate doc string", 20, 20); -return x_1; -} -} -static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___closed__1; -x_2 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___closed__2; -x_2 = l_Lean_MessageData_ofFormat(x_1); -return x_2; +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; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___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) { -_start: -{ -uint8_t x_9; -x_9 = lean_usize_dec_lt(x_4, x_3); -if (x_9 == 0) -{ -lean_object* x_10; -lean_dec(x_7); -lean_dec(x_2); -lean_dec(x_1); -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_5); -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; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; lean_object* x_30; lean_object* x_31; -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_unsigned_to_nat(2u); -x_15 = l_Lean_Syntax_getArg(x_11, x_14); -x_16 = l_Lean_Elab_Command_getRef(x_6, x_7, x_8); -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_replaceRef(x_11, x_17); -lean_dec(x_17); -x_20 = lean_ctor_get(x_6, 0); -x_21 = lean_ctor_get(x_6, 1); -x_22 = lean_ctor_get(x_6, 2); -x_23 = lean_ctor_get(x_6, 3); -x_24 = lean_ctor_get(x_6, 4); -x_25 = lean_ctor_get(x_6, 5); -x_26 = lean_ctor_get(x_6, 7); -x_27 = lean_ctor_get(x_6, 8); -x_28 = lean_ctor_get(x_6, 9); -x_29 = lean_ctor_get_uint8(x_6, sizeof(void*)*10); -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); -lean_inc(x_20); -x_30 = lean_alloc_ctor(0, 10, 1); -lean_ctor_set(x_30, 0, x_20); -lean_ctor_set(x_30, 1, x_21); -lean_ctor_set(x_30, 2, x_22); -lean_ctor_set(x_30, 3, x_23); -lean_ctor_set(x_30, 4, x_24); -lean_ctor_set(x_30, 5, x_25); -lean_ctor_set(x_30, 6, x_19); -lean_ctor_set(x_30, 7, x_26); -lean_ctor_set(x_30, 8, x_27); -lean_ctor_set(x_30, 9, x_28); -lean_ctor_set_uint8(x_30, sizeof(void*)*10, x_29); -lean_inc(x_30); -x_31 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1(x_15, x_30, x_7, x_18); -lean_dec(x_15); -if (lean_obj_tag(x_31) == 0) -{ -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_32 = lean_ctor_get(x_31, 0); -lean_inc(x_32); -x_33 = lean_ctor_get(x_31, 1); -lean_inc(x_33); -lean_dec(x_31); -lean_inc(x_1); -lean_inc(x_2); -lean_inc(x_11); -x_34 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__3___boxed), 8, 3); -lean_closure_set(x_34, 0, x_11); -lean_closure_set(x_34, 1, x_2); -lean_closure_set(x_34, 2, x_1); -x_35 = l_Lean_Syntax_getArg(x_11, x_12); -x_36 = l_Lean_Syntax_getOptional_x3f(x_35); -lean_dec(x_35); -if (lean_obj_tag(x_36) == 0) -{ -lean_object* x_37; lean_object* x_38; -lean_dec(x_34); -x_37 = lean_box(0); -lean_inc(x_2); -x_38 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__3(x_11, x_2, x_1, x_32, x_37, x_30, x_7, x_33); -if (lean_obj_tag(x_38) == 0) -{ -lean_object* x_39; lean_object* x_40; size_t x_41; size_t 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 = 1; -x_42 = lean_usize_add(x_4, x_41); -x_43 = lean_array_uset(x_13, x_4, x_39); -x_4 = x_42; -x_5 = x_43; -x_8 = x_40; -goto _start; } else { -uint8_t x_45; -lean_dec(x_13); +uint8_t x_39; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_45 = !lean_is_exclusive(x_38); -if (x_45 == 0) +x_39 = !lean_is_exclusive(x_22); +if (x_39 == 0) { -return x_38; +return x_22; } else { -lean_object* x_46; lean_object* x_47; lean_object* x_48; -x_46 = lean_ctor_get(x_38, 0); -x_47 = lean_ctor_get(x_38, 1); -lean_inc(x_47); -lean_inc(x_46); -lean_dec(x_38); -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_40; lean_object* x_41; lean_object* x_42; +x_40 = lean_ctor_get(x_22, 0); +x_41 = lean_ctor_get(x_22, 1); +lean_inc(x_41); +lean_inc(x_40); +lean_dec(x_22); +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_49; +uint8_t x_43; lean_dec(x_11); -x_49 = lean_ctor_get(x_32, 0); -lean_inc(x_49); -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_36, 0); -lean_inc(x_50); -lean_dec(x_36); -x_51 = lean_box(0); -lean_inc(x_7); -x_52 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__4(x_50, x_34, x_32, x_51, x_30, x_7, x_33); -lean_dec(x_50); -if (lean_obj_tag(x_52) == 0) -{ -lean_object* x_53; lean_object* x_54; size_t x_55; size_t x_56; lean_object* x_57; -x_53 = lean_ctor_get(x_52, 0); -lean_inc(x_53); -x_54 = lean_ctor_get(x_52, 1); -lean_inc(x_54); -lean_dec(x_52); -x_55 = 1; -x_56 = lean_usize_add(x_4, x_55); -x_57 = lean_array_uset(x_13, x_4, x_53); -x_4 = x_56; -x_5 = x_57; -x_8 = x_54; -goto _start; -} -else -{ -uint8_t x_59; -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_4); lean_dec(x_2); lean_dec(x_1); -x_59 = !lean_is_exclusive(x_52); -if (x_59 == 0) +x_43 = !lean_is_exclusive(x_19); +if (x_43 == 0) { -return x_52; +return x_19; } else { -lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_60 = lean_ctor_get(x_52, 0); -x_61 = lean_ctor_get(x_52, 1); -lean_inc(x_61); -lean_inc(x_60); -lean_dec(x_52); -x_62 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_62, 0, x_60); -lean_ctor_set(x_62, 1, x_61); -return x_62; -} +lean_object* x_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 -{ -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_dec(x_49); -x_63 = lean_ctor_get(x_36, 0); -lean_inc(x_63); -lean_dec(x_36); -x_64 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___closed__3; -x_65 = 2; -lean_inc(x_30); -x_66 = l_Lean_logAt___at_Lean_Elab_Command_elabCommand___spec__4(x_63, x_64, x_65, x_30, x_7, x_33); -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_7); -x_69 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__4(x_63, x_34, x_32, x_67, x_30, x_7, x_68); -lean_dec(x_67); -lean_dec(x_63); -if (lean_obj_tag(x_69) == 0) -{ -lean_object* x_70; lean_object* x_71; size_t x_72; size_t x_73; lean_object* x_74; -x_70 = lean_ctor_get(x_69, 0); -lean_inc(x_70); -x_71 = lean_ctor_get(x_69, 1); -lean_inc(x_71); -lean_dec(x_69); -x_72 = 1; -x_73 = lean_usize_add(x_4, x_72); -x_74 = lean_array_uset(x_13, x_4, x_70); -x_4 = x_73; -x_5 = x_74; -x_8 = x_71; -goto _start; } else { -uint8_t x_76; -lean_dec(x_13); +uint8_t x_47; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_76 = !lean_is_exclusive(x_69); -if (x_76 == 0) +x_47 = !lean_is_exclusive(x_15); +if (x_47 == 0) { -return x_69; +return x_15; } else { -lean_object* x_77; lean_object* x_78; lean_object* x_79; -x_77 = lean_ctor_get(x_69, 0); -x_78 = lean_ctor_get(x_69, 1); -lean_inc(x_78); -lean_inc(x_77); -lean_dec(x_69); -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_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_80; -lean_dec(x_30); -lean_dec(x_13); +uint8_t x_51; lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_80 = !lean_is_exclusive(x_31); -if (x_80 == 0) -{ -return x_31; -} -else -{ -lean_object* x_81; lean_object* x_82; lean_object* x_83; -x_81 = lean_ctor_get(x_31, 0); -x_82 = lean_ctor_get(x_31, 1); -lean_inc(x_82); -lean_inc(x_81); -lean_dec(x_31); -x_83 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_83, 0, x_81); -lean_ctor_set(x_83, 1, x_82); -return x_83; -} -} -} -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___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) { -_start: -{ -uint8_t x_7; -x_7 = lean_usize_dec_lt(x_2, x_1); -if (x_7 == 0) +x_51 = !lean_is_exclusive(x_13); +if (x_51 == 0) { -lean_object* x_8; -x_8 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_8, 0, x_3); -lean_ctor_set(x_8, 1, x_6); -return x_8; +return x_13; } 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; lean_object* x_20; lean_object* x_21; lean_object* x_22; size_t x_23; size_t x_24; lean_object* x_25; -x_9 = lean_array_uget(x_3, x_2); -x_10 = lean_unsigned_to_nat(0u); -x_11 = lean_array_uset(x_3, x_2, x_10); -x_12 = l_Lean_Syntax_getArg(x_9, x_10); -x_13 = lean_unsigned_to_nat(1u); -x_14 = l_Lean_Syntax_getArg(x_9, x_13); -x_15 = l_Lean_Syntax_getId(x_14); -lean_dec(x_14); -x_16 = lean_unsigned_to_nat(3u); -x_17 = l_Lean_Syntax_getArg(x_9, x_16); -x_18 = lean_unsigned_to_nat(4u); -x_19 = l_Lean_Syntax_getArg(x_9, x_18); -x_20 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_20, 0, x_9); -lean_ctor_set(x_20, 1, x_12); -lean_ctor_set(x_20, 2, x_15); -lean_ctor_set(x_20, 3, x_17); -lean_ctor_set(x_20, 4, x_19); -x_21 = l_Lean_Elab_Command_getRef(x_4, x_5, x_6); -x_22 = lean_ctor_get(x_21, 1); -lean_inc(x_22); -lean_dec(x_21); -x_23 = 1; -x_24 = lean_usize_add(x_2, x_23); -x_25 = lean_array_uset(x_11, x_2, x_20); -x_2 = x_24; -x_3 = x_25; -x_6 = x_22; -goto _start; -} -} -} -static lean_object* _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("note: this linter can be disabled with `set_option ", 51, 51); -return x_1; +lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_52 = lean_ctor_get(x_13, 0); +x_53 = lean_ctor_get(x_13, 1); +lean_inc(x_53); +lean_inc(x_52); +lean_dec(x_13); +x_54 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_54, 0, x_52); +lean_ctor_set(x_54, 1, x_53); +return x_54; } } -static lean_object* _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; } } -static lean_object* _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__3() { +static lean_object* _init_l_Lean_Elab_Command_elabAxiom___lambda__4___closed__1() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked(" false`", 7, 7); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_unsigned_to_nat(10u); +x_2 = lean_unsigned_to_nat(1u); +x_3 = l_Nat_nextPowerOfTwo_go(x_1, x_2, lean_box(0)); +return x_3; } } -static lean_object* _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__4() { +static lean_object* _init_l_Lean_Elab_Command_elabAxiom___lambda__4___closed__2() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__3; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__1; +x_3 = lean_mk_array(x_2, x_1); +return x_3; } } -static lean_object* _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__5() { +static lean_object* _init_l_Lean_Elab_Command_elabAxiom___lambda__4___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("\n", 1, 1); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_unsigned_to_nat(0u); +x_2 = l_Lean_Elab_Command_elabAxiom___lambda__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_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__6() { +static lean_object* _init_l_Lean_Elab_Command_elabAxiom___lambda__4___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__5; -x_2 = l_Lean_stringToMessageData(x_1); +x_1 = lean_box(0); +x_2 = lean_array_mk(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___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: -{ -uint8_t x_7; -x_7 = !lean_is_exclusive(x_1); -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; uint8_t x_21; lean_object* x_22; -x_8 = lean_ctor_get(x_1, 0); -x_9 = lean_ctor_get(x_1, 1); -lean_dec(x_9); -lean_inc(x_8); -x_10 = l_Lean_MessageData_ofName(x_8); -x_11 = l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__2; -lean_ctor_set_tag(x_1, 7); -lean_ctor_set(x_1, 1, x_10); -lean_ctor_set(x_1, 0, x_11); -x_12 = l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__4; -x_13 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_13, 0, x_1); -lean_ctor_set(x_13, 1, x_12); -x_14 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__9; -x_15 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_15, 0, x_14); -lean_ctor_set(x_15, 1, x_3); -x_16 = l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__6; -x_17 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_17, 0, x_15); -lean_ctor_set(x_17, 1, x_16); -x_18 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_18, 0, x_17); -lean_ctor_set(x_18, 1, x_13); -x_19 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_19, 0, x_18); -lean_ctor_set(x_19, 1, x_14); -x_20 = lean_alloc_ctor(8, 2, 0); -lean_ctor_set(x_20, 0, x_8); -lean_ctor_set(x_20, 1, x_19); -x_21 = 1; -x_22 = l_Lean_logAt___at_Lean_Elab_Command_elabCommand___spec__4(x_2, x_20, x_21, x_4, x_5, x_6); -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_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; lean_object* x_37; -x_23 = lean_ctor_get(x_1, 0); -lean_inc(x_23); -lean_dec(x_1); -lean_inc(x_23); -x_24 = l_Lean_MessageData_ofName(x_23); -x_25 = l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__2; -x_26 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_26, 1, x_24); -x_27 = l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__4; -x_28 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_28, 0, x_26); -lean_ctor_set(x_28, 1, x_27); -x_29 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__9; -x_30 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_30, 0, x_29); -lean_ctor_set(x_30, 1, x_3); -x_31 = l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__6; -x_32 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_32, 0, x_30); -lean_ctor_set(x_32, 1, x_31); -x_33 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_33, 0, x_32); -lean_ctor_set(x_33, 1, x_28); -x_34 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_34, 0, x_33); -lean_ctor_set(x_34, 1, x_29); -x_35 = lean_alloc_ctor(8, 2, 0); -lean_ctor_set(x_35, 0, x_23); -lean_ctor_set(x_35, 1, x_34); -x_36 = 1; -x_37 = l_Lean_logAt___at_Lean_Elab_Command_elabCommand___spec__4(x_2, x_35, x_36, x_4, x_5, x_6); -return x_37; -} -} -} -LEAN_EXPORT lean_object* l_Lean_Linter_logLintIf___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -lean_object* x_7; uint8_t x_8; -x_7 = lean_st_ref_get(x_5, x_6); -x_8 = !lean_is_exclusive(x_7); -if (x_8 == 0) -{ -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; -x_9 = lean_ctor_get(x_7, 0); -x_10 = lean_ctor_get(x_7, 1); -x_11 = lean_ctor_get(x_9, 2); -lean_inc(x_11); -lean_dec(x_9); -x_12 = l_Lean_Elab_Command_instInhabitedScope; -x_13 = l_List_head_x21___rarg(x_12, x_11); -lean_dec(x_11); -x_14 = lean_ctor_get(x_13, 1); -lean_inc(x_14); -lean_dec(x_13); -lean_inc(x_1); -x_15 = l_Lean_Linter_getLinterValue(x_1, x_14); -lean_dec(x_14); -if (x_15 == 0) -{ -lean_object* x_16; -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_16 = lean_box(0); -lean_ctor_set(x_7, 0, x_16); -return x_7; -} -else -{ -lean_object* x_17; -lean_free_object(x_7); -x_17 = l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6(x_1, x_2, x_3, x_4, x_5, x_10); -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; uint8_t x_24; -x_18 = lean_ctor_get(x_7, 0); -x_19 = lean_ctor_get(x_7, 1); -lean_inc(x_19); -lean_inc(x_18); -lean_dec(x_7); -x_20 = lean_ctor_get(x_18, 2); -lean_inc(x_20); -lean_dec(x_18); -x_21 = l_Lean_Elab_Command_instInhabitedScope; -x_22 = l_List_head_x21___rarg(x_21, x_20); -lean_dec(x_20); -x_23 = lean_ctor_get(x_22, 1); -lean_inc(x_23); -lean_dec(x_22); -lean_inc(x_1); -x_24 = l_Lean_Linter_getLinterValue(x_1, x_23); -lean_dec(x_23); -if (x_24 == 0) -{ -lean_object* x_25; lean_object* x_26; -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -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_19); -return x_26; -} -else -{ -lean_object* x_27; -x_27 = l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6(x_1, x_2, x_3, x_4, x_5, x_19); -return x_27; -} -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___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) { +static lean_object* _init_l_Lean_Elab_Command_elabAxiom___lambda__4___closed__5() { _start: { -lean_object* x_16; lean_object* x_17; -x_16 = lean_alloc_ctor(0, 11, 0); -lean_ctor_set(x_16, 0, x_1); -lean_ctor_set(x_16, 1, x_2); -lean_ctor_set(x_16, 2, x_3); -lean_ctor_set(x_16, 3, x_4); -lean_ctor_set(x_16, 4, x_5); -lean_ctor_set(x_16, 5, x_6); -lean_ctor_set(x_16, 6, x_7); -lean_ctor_set(x_16, 7, x_8); -lean_ctor_set(x_16, 8, x_9); -lean_ctor_set(x_16, 9, x_10); -lean_ctor_set(x_16, 10, x_11); -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_16); -lean_ctor_set(x_17, 1, x_15); -return x_17; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__3; +x_2 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__4; +x_3 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_1); +lean_ctor_set(x_3, 2, x_2); +return x_3; } } -static lean_object* _init_l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1() { +static lean_object* _init_l_Lean_Elab_Command_elabAxiom___lambda__4___closed__6() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked(":=", 2, 2); +x_1 = lean_mk_string_unchecked("Elab", 4, 4); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__2() { +static lean_object* _init_l_Lean_Elab_Command_elabAxiom___lambda__4___closed__7() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("'inductive ... :=' has been deprecated in favor of 'inductive ... where'.", 73, 73); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__6; +x_2 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__14; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; } } -static lean_object* _init_l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__3() { +static lean_object* _init_l_Lean_Elab_Command_elabAxiom___lambda__4___closed__8() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__2; -x_2 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("", 0, 0); +return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__4() { +static lean_object* _init_l_Lean_Elab_Command_elabAxiom___lambda__4___closed__9() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__3; -x_2 = l_Lean_MessageData_ofFormat(x_1); +x_1 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__8; +x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__5() { +static lean_object* _init_l_Lean_Elab_Command_elabAxiom___lambda__4___closed__10() { _start: { lean_object* x_1; -x_1 = l_Lean_Linter_linter_deprecated; +x_1 = lean_mk_string_unchecked(" : ", 3, 3); return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView(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_Elab_Command_elabAxiom___lambda__4___closed__11() { _start: { -lean_object* x_6; -lean_inc(x_3); -x_6 = l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1(x_1, x_3, x_4, x_5); -if (lean_obj_tag(x_6) == 0) +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__10; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +_start: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_7 = lean_ctor_get(x_6, 1); -lean_inc(x_7); -lean_dec(x_6); -x_8 = lean_unsigned_to_nat(2u); -x_9 = l_Lean_Syntax_getArg(x_2, x_8); -x_10 = l_Lean_Elab_expandOptDeclSig(x_9); -lean_dec(x_9); -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -x_12 = lean_ctor_get(x_10, 1); +lean_object* x_17; uint8_t x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_1, 2); +lean_inc(x_17); +x_18 = 2; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); lean_inc(x_12); -lean_dec(x_10); -x_13 = lean_unsigned_to_nat(1u); -x_14 = l_Lean_Syntax_getArg(x_2, x_13); -lean_inc(x_3); -lean_inc(x_1); -x_15 = l_Lean_Elab_Command_expandDeclId(x_14, x_1, x_3, x_4, x_7); -if (lean_obj_tag(x_15) == 0) -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; size_t x_26; size_t x_27; lean_object* x_28; -x_16 = lean_ctor_get(x_15, 0); -lean_inc(x_16); -x_17 = lean_ctor_get(x_15, 1); +lean_inc(x_11); +lean_inc(x_10); lean_inc(x_17); -lean_dec(x_15); -x_18 = lean_ctor_get(x_16, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_16, 1); -lean_inc(x_19); -x_20 = lean_ctor_get(x_16, 2); -lean_inc(x_20); -lean_dec(x_16); -lean_inc(x_3); lean_inc(x_2); -lean_inc(x_19); -x_21 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1(x_19, x_2, x_3, x_4, x_17); -x_22 = lean_ctor_get(x_21, 1); +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); +if (lean_obj_tag(x_19) == 0) +{ +lean_object* x_20; lean_object* x_21; +x_20 = lean_ctor_get(x_19, 1); +lean_inc(x_20); +lean_dec(x_19); +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_21 = l_Lean_Elab_Term_elabType(x_3, x_10, x_11, x_12, x_13, x_14, x_15, x_20); +if (lean_obj_tag(x_21) == 0) +{ +lean_object* x_22; lean_object* x_23; uint8_t 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_23 = lean_unsigned_to_nat(4u); -x_24 = l_Lean_Syntax_getArg(x_2, x_23); -x_25 = l_Lean_Syntax_getArgs(x_24); -lean_dec(x_24); -x_26 = lean_array_size(x_25); -x_27 = 0; -lean_inc(x_4); -lean_inc(x_19); -lean_inc(x_1); -x_28 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3(x_1, x_19, x_26, x_27, x_25, x_3, x_4, x_22); +x_24 = 1; +x_25 = 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_26 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_24, x_25, x_10, x_11, x_12, x_13, x_14, x_15, x_23); +if (lean_obj_tag(x_26) == 0) +{ +lean_object* x_27; lean_object* x_28; +x_27 = lean_ctor_get(x_26, 1); +lean_inc(x_27); +lean_dec(x_26); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_10); +x_28 = l_Lean_Elab_Term_addAutoBoundImplicits(x_9, 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; lean_object* x_33; lean_object* x_34; +lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; x_29 = lean_ctor_get(x_28, 0); lean_inc(x_29); x_30 = lean_ctor_get(x_28, 1); lean_inc(x_30); lean_dec(x_28); -x_31 = lean_unsigned_to_nat(5u); -x_32 = l_Lean_Syntax_getArg(x_2, x_31); -x_33 = l_Lean_Syntax_getOptional_x3f(x_32); -lean_dec(x_32); -if (lean_obj_tag(x_33) == 0) -{ -lean_object* x_80; -x_80 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__4; -x_34 = x_80; -goto block_79; -} -else +x_31 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_22, x_10, x_11, x_12, x_13, x_14, x_15, x_30); +x_32 = !lean_is_exclusive(x_31); +if (x_32 == 0) { -lean_object* x_81; lean_object* x_82; lean_object* x_83; -x_81 = lean_ctor_get(x_33, 0); -lean_inc(x_81); -lean_dec(x_33); -x_82 = l_Lean_Syntax_getArg(x_81, x_13); -lean_dec(x_81); -x_83 = l_Lean_Syntax_getArgs(x_82); -lean_dec(x_82); -x_34 = x_83; -goto block_79; -} -block_79: +lean_object* x_33; lean_object* x_34; uint8_t x_35; uint8_t x_36; lean_object* x_37; +x_33 = lean_ctor_get(x_31, 0); +x_34 = lean_ctor_get(x_31, 1); +x_35 = 1; +x_36 = 1; +x_37 = l_Lean_Meta_mkForallFVars(x_29, x_33, x_25, x_35, x_36, x_12, x_13, x_14, x_15, x_34); +if (lean_obj_tag(x_37) == 0) { -size_t x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_35 = lean_array_size(x_34); -x_36 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__4(x_35, x_27, x_34, x_3, x_4, x_30); -x_37 = lean_ctor_get(x_36, 0); -lean_inc(x_37); -x_38 = lean_ctor_get(x_36, 1); +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_37, 0); lean_inc(x_38); -lean_dec(x_36); -x_39 = lean_unsigned_to_nat(6u); -x_40 = l_Lean_Syntax_getArg(x_2, x_39); -x_41 = lean_alloc_closure((void*)(l_Lean_Elab_getOptDerivingClasses), 4, 1); -lean_closure_set(x_41, 0, x_40); -x_42 = l_Lean_Elab_Command_liftCoreM___rarg(x_41, x_3, x_4, x_38); -if (lean_obj_tag(x_42) == 0) -{ -lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; uint8_t x_50; -x_43 = lean_ctor_get(x_42, 0); -lean_inc(x_43); -x_44 = lean_ctor_get(x_42, 1); -lean_inc(x_44); -lean_dec(x_42); -x_45 = lean_unsigned_to_nat(3u); -x_46 = l_Lean_Syntax_getArg(x_2, x_45); -x_47 = lean_unsigned_to_nat(0u); -x_48 = l_Lean_Syntax_getArg(x_46, x_47); -x_49 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1; -x_50 = l_Lean_Syntax_isToken(x_49, x_48); -lean_dec(x_48); -if (x_50 == 0) +x_39 = lean_ctor_get(x_37, 1); +lean_inc(x_39); +lean_dec(x_37); +x_40 = l_Lean_Meta_mkForallFVars(x_4, x_38, x_35, x_35, x_36, x_12, x_13, x_14, x_15, x_39); +if (lean_obj_tag(x_40) == 0) +{ +lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; uint8_t x_45; +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___private_Lean_Elab_Declaration_0__Lean_Elab_Command_ensureValidNamespace___closed__2; +x_44 = l_Lean_Elab_Term_levelMVarToParam(x_41, x_43, x_10, x_11, x_12, x_13, x_14, x_15, x_42); +x_45 = !lean_is_exclusive(x_44); +if (x_45 == 0) { -lean_object* x_51; lean_object* x_52; +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_46 = lean_ctor_get(x_44, 0); +x_47 = lean_ctor_get(x_44, 1); +x_48 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__5; +lean_inc(x_46); +x_49 = l_Lean_CollectLevelParams_main(x_46, x_48); +x_50 = lean_ctor_get(x_49, 2); +lean_inc(x_50); +lean_dec(x_49); +x_51 = l_Lean_Elab_sortDeclLevelParams(x_5, x_6, x_50); +if (lean_obj_tag(x_51) == 0) +{ +uint8_t x_52; +lean_free_object(x_44); lean_dec(x_46); -x_51 = lean_box(0); -x_52 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___lambda__1(x_2, x_14, x_1, x_18, x_19, x_20, x_11, x_12, x_29, x_43, x_37, x_51, x_3, x_4, x_44); -lean_dec(x_4); -lean_dec(x_3); -return x_52; +lean_free_object(x_31); +lean_dec(x_17); +lean_dec(x_8); +lean_dec(x_2); +lean_dec(x_1); +x_52 = !lean_is_exclusive(x_51); +if (x_52 == 0) +{ +lean_object* x_53; lean_object* x_54; +lean_ctor_set_tag(x_51, 3); +x_53 = l_Lean_MessageData_ofFormat(x_51); +x_54 = l_Lean_throwErrorAt___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__12(x_7, x_53, x_10, x_11, x_12, x_13, x_14, x_15, x_47); +lean_dec(x_15); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +return x_54; } else { -lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; uint8_t x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; -x_53 = l_Lean_Syntax_getArg(x_2, x_47); -x_54 = l_Lean_Elab_Command_getRef(x_3, x_4, x_44); -x_55 = lean_ctor_get(x_54, 0); +lean_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); -x_56 = lean_ctor_get(x_54, 1); -lean_inc(x_56); -lean_dec(x_54); -x_57 = l_Lean_replaceRef(x_53, x_55); -lean_dec(x_55); -lean_dec(x_53); -x_58 = lean_ctor_get(x_3, 0); -lean_inc(x_58); -x_59 = lean_ctor_get(x_3, 1); -lean_inc(x_59); -x_60 = lean_ctor_get(x_3, 2); -lean_inc(x_60); -x_61 = lean_ctor_get(x_3, 3); -lean_inc(x_61); -x_62 = lean_ctor_get(x_3, 4); -lean_inc(x_62); -x_63 = lean_ctor_get(x_3, 5); +lean_dec(x_51); +x_56 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_56, 0, x_55); +x_57 = l_Lean_MessageData_ofFormat(x_56); +x_58 = l_Lean_throwErrorAt___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__12(x_7, x_57, x_10, x_11, x_12, x_13, x_14, x_15, x_47); +lean_dec(x_15); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +return x_58; +} +} +else +{ +uint8_t x_59; +x_59 = !lean_is_exclusive(x_51); +if (x_59 == 0) +{ +lean_object* x_60; lean_object* x_61; uint8_t x_62; +x_60 = lean_ctor_get(x_51, 0); +x_61 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_46, x_10, x_11, x_12, x_13, x_14, x_15, x_47); +x_62 = !lean_is_exclusive(x_61); +if (x_62 == 0) +{ +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; uint8_t x_71; +x_63 = lean_ctor_get(x_61, 0); +x_64 = lean_ctor_get(x_61, 1); lean_inc(x_63); -x_64 = lean_ctor_get(x_3, 7); -lean_inc(x_64); -x_65 = lean_ctor_get(x_3, 8); -lean_inc(x_65); -x_66 = lean_ctor_get(x_3, 9); -lean_inc(x_66); -x_67 = lean_ctor_get_uint8(x_3, sizeof(void*)*10); -x_68 = lean_alloc_ctor(0, 10, 1); -lean_ctor_set(x_68, 0, x_58); -lean_ctor_set(x_68, 1, x_59); -lean_ctor_set(x_68, 2, x_60); -lean_ctor_set(x_68, 3, x_61); -lean_ctor_set(x_68, 4, x_62); -lean_ctor_set(x_68, 5, x_63); -lean_ctor_set(x_68, 6, x_57); -lean_ctor_set(x_68, 7, x_64); -lean_ctor_set(x_68, 8, x_65); -lean_ctor_set(x_68, 9, x_66); -lean_ctor_set_uint8(x_68, sizeof(void*)*10, x_67); -x_69 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__5; -x_70 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__4; -x_71 = l_Lean_Linter_logLintIf___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5(x_69, x_46, x_70, x_68, x_4, x_56); -lean_dec(x_46); -x_72 = lean_ctor_get(x_71, 0); +lean_inc(x_2); +x_65 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_65, 0, x_2); +lean_ctor_set(x_65, 1, x_60); +lean_ctor_set(x_65, 2, x_63); +x_66 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 3); +lean_dec(x_1); +x_67 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_67, 0, x_65); +lean_ctor_set_uint8(x_67, sizeof(void*)*1, x_66); +lean_ctor_set_tag(x_51, 0); +lean_ctor_set(x_51, 0, x_67); +x_68 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__7; +x_69 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_68, x_10, x_11, x_12, x_13, x_14, x_15, x_64); +x_70 = lean_ctor_get(x_69, 0); +lean_inc(x_70); +x_71 = lean_unbox(x_70); +lean_dec(x_70); +if (x_71 == 0) +{ +lean_object* x_72; lean_object* x_73; lean_object* x_74; +lean_free_object(x_61); +lean_dec(x_63); +lean_free_object(x_44); +lean_free_object(x_31); +x_72 = lean_ctor_get(x_69, 1); lean_inc(x_72); -x_73 = lean_ctor_get(x_71, 1); -lean_inc(x_73); -lean_dec(x_71); -x_74 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___lambda__1(x_2, x_14, x_1, x_18, x_19, x_20, x_11, x_12, x_29, x_43, x_37, x_72, x_3, x_4, x_73); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_72); +lean_dec(x_69); +x_73 = lean_box(0); +x_74 = l_Lean_Elab_Command_elabAxiom___lambda__3(x_51, x_2, x_8, x_17, x_73, x_10, x_11, x_12, x_13, x_14, x_15, x_72); return x_74; } -} else { uint8_t x_75; -lean_dec(x_37); -lean_dec(x_29); -lean_dec(x_20); -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_14); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_4); -lean_dec(x_3); +x_75 = !lean_is_exclusive(x_69); +if (x_75 == 0) +{ +lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; +x_76 = lean_ctor_get(x_69, 1); +x_77 = lean_ctor_get(x_69, 0); +lean_dec(x_77); +lean_inc(x_2); +x_78 = l_Lean_MessageData_ofName(x_2); +x_79 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__9; +lean_ctor_set_tag(x_69, 7); +lean_ctor_set(x_69, 1, x_78); +lean_ctor_set(x_69, 0, x_79); +x_80 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__11; +lean_ctor_set_tag(x_61, 7); +lean_ctor_set(x_61, 1, x_80); +lean_ctor_set(x_61, 0, x_69); +x_81 = l_Lean_MessageData_ofExpr(x_63); +lean_ctor_set_tag(x_44, 7); +lean_ctor_set(x_44, 1, x_81); +lean_ctor_set(x_44, 0, x_61); +lean_ctor_set_tag(x_31, 7); +lean_ctor_set(x_31, 1, x_79); +lean_ctor_set(x_31, 0, x_44); +x_82 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_68, x_31, x_10, x_11, x_12, x_13, x_14, x_15, x_76); +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 = l_Lean_Elab_Command_elabAxiom___lambda__3(x_51, x_2, x_8, x_17, x_83, x_10, x_11, x_12, x_13, x_14, x_15, x_84); +lean_dec(x_83); +return x_85; +} +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; +x_86 = lean_ctor_get(x_69, 1); +lean_inc(x_86); +lean_dec(x_69); +lean_inc(x_2); +x_87 = l_Lean_MessageData_ofName(x_2); +x_88 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__9; +x_89 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_89, 0, x_88); +lean_ctor_set(x_89, 1, x_87); +x_90 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__11; +lean_ctor_set_tag(x_61, 7); +lean_ctor_set(x_61, 1, x_90); +lean_ctor_set(x_61, 0, x_89); +x_91 = l_Lean_MessageData_ofExpr(x_63); +lean_ctor_set_tag(x_44, 7); +lean_ctor_set(x_44, 1, x_91); +lean_ctor_set(x_44, 0, x_61); +lean_ctor_set_tag(x_31, 7); +lean_ctor_set(x_31, 1, x_88); +lean_ctor_set(x_31, 0, x_44); +x_92 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_68, x_31, x_10, x_11, x_12, x_13, x_14, x_15, x_86); +x_93 = lean_ctor_get(x_92, 0); +lean_inc(x_93); +x_94 = lean_ctor_get(x_92, 1); +lean_inc(x_94); +lean_dec(x_92); +x_95 = l_Lean_Elab_Command_elabAxiom___lambda__3(x_51, x_2, x_8, x_17, x_93, x_10, x_11, x_12, x_13, x_14, x_15, x_94); +lean_dec(x_93); +return x_95; +} +} +} +else +{ +lean_object* x_96; 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; +x_96 = lean_ctor_get(x_61, 0); +x_97 = lean_ctor_get(x_61, 1); +lean_inc(x_97); +lean_inc(x_96); +lean_dec(x_61); +lean_inc(x_96); +lean_inc(x_2); +x_98 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_98, 0, x_2); +lean_ctor_set(x_98, 1, x_60); +lean_ctor_set(x_98, 2, x_96); +x_99 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 3); +lean_dec(x_1); +x_100 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_100, 0, x_98); +lean_ctor_set_uint8(x_100, sizeof(void*)*1, x_99); +lean_ctor_set_tag(x_51, 0); +lean_ctor_set(x_51, 0, x_100); +x_101 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__7; +x_102 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_101, x_10, x_11, x_12, x_13, x_14, x_15, x_97); +x_103 = lean_ctor_get(x_102, 0); +lean_inc(x_103); +x_104 = lean_unbox(x_103); +lean_dec(x_103); +if (x_104 == 0) +{ +lean_object* x_105; lean_object* x_106; lean_object* x_107; +lean_dec(x_96); +lean_free_object(x_44); +lean_free_object(x_31); +x_105 = lean_ctor_get(x_102, 1); +lean_inc(x_105); +lean_dec(x_102); +x_106 = lean_box(0); +x_107 = l_Lean_Elab_Command_elabAxiom___lambda__3(x_51, x_2, x_8, x_17, x_106, x_10, x_11, x_12, x_13, x_14, x_15, x_105); +return x_107; +} +else +{ +lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; +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; +} else { + lean_dec_ref(x_102); + x_109 = lean_box(0); +} +lean_inc(x_2); +x_110 = l_Lean_MessageData_ofName(x_2); +x_111 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__9; +if (lean_is_scalar(x_109)) { + x_112 = lean_alloc_ctor(7, 2, 0); +} else { + x_112 = x_109; + lean_ctor_set_tag(x_112, 7); +} +lean_ctor_set(x_112, 0, x_111); +lean_ctor_set(x_112, 1, x_110); +x_113 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__11; +x_114 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_114, 0, x_112); +lean_ctor_set(x_114, 1, x_113); +x_115 = l_Lean_MessageData_ofExpr(x_96); +lean_ctor_set_tag(x_44, 7); +lean_ctor_set(x_44, 1, x_115); +lean_ctor_set(x_44, 0, x_114); +lean_ctor_set_tag(x_31, 7); +lean_ctor_set(x_31, 1, x_111); +lean_ctor_set(x_31, 0, x_44); +x_116 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_101, x_31, x_10, x_11, x_12, x_13, x_14, x_15, x_108); +x_117 = lean_ctor_get(x_116, 0); +lean_inc(x_117); +x_118 = lean_ctor_get(x_116, 1); +lean_inc(x_118); +lean_dec(x_116); +x_119 = l_Lean_Elab_Command_elabAxiom___lambda__3(x_51, x_2, x_8, x_17, x_117, x_10, x_11, x_12, x_13, x_14, x_15, x_118); +lean_dec(x_117); +return x_119; +} +} +} +else +{ +lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; uint8_t x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; uint8_t x_132; +x_120 = lean_ctor_get(x_51, 0); +lean_inc(x_120); +lean_dec(x_51); +x_121 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_46, x_10, x_11, x_12, x_13, x_14, x_15, x_47); +x_122 = lean_ctor_get(x_121, 0); +lean_inc(x_122); +x_123 = lean_ctor_get(x_121, 1); +lean_inc(x_123); +if (lean_is_exclusive(x_121)) { + lean_ctor_release(x_121, 0); + lean_ctor_release(x_121, 1); + x_124 = x_121; +} else { + lean_dec_ref(x_121); + x_124 = lean_box(0); +} +lean_inc(x_122); +lean_inc(x_2); +x_125 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_125, 0, x_2); +lean_ctor_set(x_125, 1, x_120); +lean_ctor_set(x_125, 2, x_122); +x_126 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 3); +lean_dec(x_1); +x_127 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_127, 0, x_125); +lean_ctor_set_uint8(x_127, sizeof(void*)*1, x_126); +x_128 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_128, 0, x_127); +x_129 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__7; +x_130 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_129, x_10, x_11, x_12, x_13, x_14, x_15, x_123); +x_131 = lean_ctor_get(x_130, 0); +lean_inc(x_131); +x_132 = lean_unbox(x_131); +lean_dec(x_131); +if (x_132 == 0) +{ +lean_object* x_133; lean_object* x_134; lean_object* x_135; +lean_dec(x_124); +lean_dec(x_122); +lean_free_object(x_44); +lean_free_object(x_31); +x_133 = lean_ctor_get(x_130, 1); +lean_inc(x_133); +lean_dec(x_130); +x_134 = lean_box(0); +x_135 = l_Lean_Elab_Command_elabAxiom___lambda__3(x_128, x_2, x_8, x_17, x_134, x_10, x_11, x_12, x_13, x_14, x_15, x_133); +return x_135; +} +else +{ +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_136 = lean_ctor_get(x_130, 1); +lean_inc(x_136); +if (lean_is_exclusive(x_130)) { + lean_ctor_release(x_130, 0); + lean_ctor_release(x_130, 1); + x_137 = x_130; +} else { + lean_dec_ref(x_130); + x_137 = lean_box(0); +} +lean_inc(x_2); +x_138 = l_Lean_MessageData_ofName(x_2); +x_139 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__9; +if (lean_is_scalar(x_137)) { + x_140 = lean_alloc_ctor(7, 2, 0); +} else { + x_140 = x_137; + lean_ctor_set_tag(x_140, 7); +} +lean_ctor_set(x_140, 0, x_139); +lean_ctor_set(x_140, 1, x_138); +x_141 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__11; +if (lean_is_scalar(x_124)) { + x_142 = lean_alloc_ctor(7, 2, 0); +} else { + x_142 = x_124; + lean_ctor_set_tag(x_142, 7); +} +lean_ctor_set(x_142, 0, x_140); +lean_ctor_set(x_142, 1, x_141); +x_143 = l_Lean_MessageData_ofExpr(x_122); +lean_ctor_set_tag(x_44, 7); +lean_ctor_set(x_44, 1, x_143); +lean_ctor_set(x_44, 0, x_142); +lean_ctor_set_tag(x_31, 7); +lean_ctor_set(x_31, 1, x_139); +lean_ctor_set(x_31, 0, x_44); +x_144 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_129, x_31, x_10, x_11, x_12, x_13, x_14, x_15, 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 = l_Lean_Elab_Command_elabAxiom___lambda__3(x_128, x_2, x_8, x_17, x_145, x_10, x_11, x_12, x_13, x_14, x_15, x_146); +lean_dec(x_145); +return x_147; +} +} +} +} +else +{ +lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; +x_148 = lean_ctor_get(x_44, 0); +x_149 = lean_ctor_get(x_44, 1); +lean_inc(x_149); +lean_inc(x_148); +lean_dec(x_44); +x_150 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__5; +lean_inc(x_148); +x_151 = l_Lean_CollectLevelParams_main(x_148, x_150); +x_152 = lean_ctor_get(x_151, 2); +lean_inc(x_152); +lean_dec(x_151); +x_153 = l_Lean_Elab_sortDeclLevelParams(x_5, x_6, x_152); +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_dec(x_148); +lean_free_object(x_31); +lean_dec(x_17); +lean_dec(x_8); lean_dec(x_2); lean_dec(x_1); -x_75 = !lean_is_exclusive(x_42); -if (x_75 == 0) +x_154 = lean_ctor_get(x_153, 0); +lean_inc(x_154); +if (lean_is_exclusive(x_153)) { + lean_ctor_release(x_153, 0); + x_155 = x_153; +} else { + lean_dec_ref(x_153); + x_155 = lean_box(0); +} +if (lean_is_scalar(x_155)) { + x_156 = lean_alloc_ctor(3, 1, 0); +} else { + x_156 = x_155; + lean_ctor_set_tag(x_156, 3); +} +lean_ctor_set(x_156, 0, x_154); +x_157 = l_Lean_MessageData_ofFormat(x_156); +x_158 = l_Lean_throwErrorAt___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__12(x_7, x_157, x_10, x_11, x_12, x_13, x_14, x_15, x_149); +lean_dec(x_15); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +return x_158; +} +else { -return x_42; +lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; uint8_t x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; uint8_t x_172; +x_159 = lean_ctor_get(x_153, 0); +lean_inc(x_159); +if (lean_is_exclusive(x_153)) { + lean_ctor_release(x_153, 0); + x_160 = x_153; +} else { + lean_dec_ref(x_153); + x_160 = lean_box(0); +} +x_161 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_148, x_10, x_11, x_12, x_13, x_14, x_15, x_149); +x_162 = lean_ctor_get(x_161, 0); +lean_inc(x_162); +x_163 = lean_ctor_get(x_161, 1); +lean_inc(x_163); +if (lean_is_exclusive(x_161)) { + lean_ctor_release(x_161, 0); + lean_ctor_release(x_161, 1); + x_164 = x_161; +} else { + lean_dec_ref(x_161); + x_164 = lean_box(0); +} +lean_inc(x_162); +lean_inc(x_2); +x_165 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_165, 0, x_2); +lean_ctor_set(x_165, 1, x_159); +lean_ctor_set(x_165, 2, x_162); +x_166 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 3); +lean_dec(x_1); +x_167 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_167, 0, x_165); +lean_ctor_set_uint8(x_167, sizeof(void*)*1, x_166); +if (lean_is_scalar(x_160)) { + x_168 = lean_alloc_ctor(0, 1, 0); +} else { + x_168 = x_160; + lean_ctor_set_tag(x_168, 0); +} +lean_ctor_set(x_168, 0, x_167); +x_169 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__7; +x_170 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_169, x_10, x_11, x_12, x_13, x_14, x_15, x_163); +x_171 = lean_ctor_get(x_170, 0); +lean_inc(x_171); +x_172 = lean_unbox(x_171); +lean_dec(x_171); +if (x_172 == 0) +{ +lean_object* x_173; lean_object* x_174; lean_object* x_175; +lean_dec(x_164); +lean_dec(x_162); +lean_free_object(x_31); +x_173 = lean_ctor_get(x_170, 1); +lean_inc(x_173); +lean_dec(x_170); +x_174 = lean_box(0); +x_175 = l_Lean_Elab_Command_elabAxiom___lambda__3(x_168, x_2, x_8, x_17, x_174, x_10, x_11, x_12, x_13, x_14, x_15, x_173); +return x_175; } else { -lean_object* x_76; lean_object* x_77; lean_object* x_78; -x_76 = lean_ctor_get(x_42, 0); -x_77 = lean_ctor_get(x_42, 1); -lean_inc(x_77); -lean_inc(x_76); -lean_dec(x_42); -x_78 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_78, 0, x_76); -lean_ctor_set(x_78, 1, x_77); -return x_78; +lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; +x_176 = lean_ctor_get(x_170, 1); +lean_inc(x_176); +if (lean_is_exclusive(x_170)) { + lean_ctor_release(x_170, 0); + lean_ctor_release(x_170, 1); + x_177 = x_170; +} else { + lean_dec_ref(x_170); + x_177 = lean_box(0); +} +lean_inc(x_2); +x_178 = l_Lean_MessageData_ofName(x_2); +x_179 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__9; +if (lean_is_scalar(x_177)) { + x_180 = lean_alloc_ctor(7, 2, 0); +} else { + x_180 = x_177; + lean_ctor_set_tag(x_180, 7); +} +lean_ctor_set(x_180, 0, x_179); +lean_ctor_set(x_180, 1, x_178); +x_181 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__11; +if (lean_is_scalar(x_164)) { + x_182 = lean_alloc_ctor(7, 2, 0); +} else { + x_182 = x_164; + lean_ctor_set_tag(x_182, 7); +} +lean_ctor_set(x_182, 0, x_180); +lean_ctor_set(x_182, 1, x_181); +x_183 = l_Lean_MessageData_ofExpr(x_162); +x_184 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_184, 0, x_182); +lean_ctor_set(x_184, 1, x_183); +lean_ctor_set_tag(x_31, 7); +lean_ctor_set(x_31, 1, x_179); +lean_ctor_set(x_31, 0, x_184); +x_185 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_169, x_31, x_10, x_11, x_12, x_13, x_14, x_15, x_176); +x_186 = lean_ctor_get(x_185, 0); +lean_inc(x_186); +x_187 = lean_ctor_get(x_185, 1); +lean_inc(x_187); +lean_dec(x_185); +x_188 = l_Lean_Elab_Command_elabAxiom___lambda__3(x_168, x_2, x_8, x_17, x_186, x_10, x_11, x_12, x_13, x_14, x_15, x_187); +lean_dec(x_186); +return x_188; } } } } else { -uint8_t x_84; -lean_dec(x_20); -lean_dec(x_19); -lean_dec(x_18); +uint8_t x_189; +lean_free_object(x_31); +lean_dec(x_17); +lean_dec(x_15); lean_dec(x_14); +lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); -lean_dec(x_4); -lean_dec(x_3); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_5); lean_dec(x_2); lean_dec(x_1); -x_84 = !lean_is_exclusive(x_28); -if (x_84 == 0) +x_189 = !lean_is_exclusive(x_40); +if (x_189 == 0) { -return x_28; +return x_40; } else { -lean_object* x_85; lean_object* x_86; lean_object* x_87; -x_85 = lean_ctor_get(x_28, 0); -x_86 = lean_ctor_get(x_28, 1); -lean_inc(x_86); -lean_inc(x_85); -lean_dec(x_28); -x_87 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_87, 0, x_85); -lean_ctor_set(x_87, 1, x_86); -return x_87; +lean_object* x_190; lean_object* x_191; lean_object* x_192; +x_190 = lean_ctor_get(x_40, 0); +x_191 = lean_ctor_get(x_40, 1); +lean_inc(x_191); +lean_inc(x_190); +lean_dec(x_40); +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; } } } else { -uint8_t x_88; +uint8_t x_193; +lean_free_object(x_31); +lean_dec(x_17); +lean_dec(x_15); lean_dec(x_14); +lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_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_88 = !lean_is_exclusive(x_15); -if (x_88 == 0) +x_193 = !lean_is_exclusive(x_37); +if (x_193 == 0) { -return x_15; +return x_37; } else { -lean_object* x_89; lean_object* x_90; lean_object* x_91; -x_89 = lean_ctor_get(x_15, 0); -x_90 = lean_ctor_get(x_15, 1); -lean_inc(x_90); -lean_inc(x_89); -lean_dec(x_15); -x_91 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_91, 0, x_89); -lean_ctor_set(x_91, 1, x_90); -return x_91; +lean_object* x_194; lean_object* x_195; lean_object* x_196; +x_194 = lean_ctor_get(x_37, 0); +x_195 = lean_ctor_get(x_37, 1); +lean_inc(x_195); +lean_inc(x_194); +lean_dec(x_37); +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_92; -lean_dec(x_4); -lean_dec(x_3); +lean_object* x_197; lean_object* x_198; uint8_t x_199; uint8_t x_200; lean_object* x_201; +x_197 = lean_ctor_get(x_31, 0); +x_198 = lean_ctor_get(x_31, 1); +lean_inc(x_198); +lean_inc(x_197); +lean_dec(x_31); +x_199 = 1; +x_200 = 1; +x_201 = l_Lean_Meta_mkForallFVars(x_29, x_197, x_25, x_199, x_200, x_12, x_13, x_14, x_15, x_198); +if (lean_obj_tag(x_201) == 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); +lean_dec(x_201); +x_204 = l_Lean_Meta_mkForallFVars(x_4, x_202, x_199, x_199, x_200, x_12, x_13, x_14, x_15, x_203); +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; +x_205 = lean_ctor_get(x_204, 0); +lean_inc(x_205); +x_206 = lean_ctor_get(x_204, 1); +lean_inc(x_206); +lean_dec(x_204); +x_207 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_ensureValidNamespace___closed__2; +x_208 = l_Lean_Elab_Term_levelMVarToParam(x_205, x_207, x_10, x_11, x_12, x_13, x_14, x_15, x_206); +x_209 = lean_ctor_get(x_208, 0); +lean_inc(x_209); +x_210 = lean_ctor_get(x_208, 1); +lean_inc(x_210); +if (lean_is_exclusive(x_208)) { + lean_ctor_release(x_208, 0); + lean_ctor_release(x_208, 1); + x_211 = x_208; +} else { + lean_dec_ref(x_208); + x_211 = lean_box(0); +} +x_212 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__5; +lean_inc(x_209); +x_213 = l_Lean_CollectLevelParams_main(x_209, x_212); +x_214 = lean_ctor_get(x_213, 2); +lean_inc(x_214); +lean_dec(x_213); +x_215 = l_Lean_Elab_sortDeclLevelParams(x_5, x_6, x_214); +if (lean_obj_tag(x_215) == 0) +{ +lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; +lean_dec(x_211); +lean_dec(x_209); +lean_dec(x_17); +lean_dec(x_8); lean_dec(x_2); lean_dec(x_1); -x_92 = !lean_is_exclusive(x_6); -if (x_92 == 0) +x_216 = lean_ctor_get(x_215, 0); +lean_inc(x_216); +if (lean_is_exclusive(x_215)) { + lean_ctor_release(x_215, 0); + x_217 = x_215; +} else { + lean_dec_ref(x_215); + x_217 = lean_box(0); +} +if (lean_is_scalar(x_217)) { + x_218 = lean_alloc_ctor(3, 1, 0); +} else { + x_218 = x_217; + lean_ctor_set_tag(x_218, 3); +} +lean_ctor_set(x_218, 0, x_216); +x_219 = l_Lean_MessageData_ofFormat(x_218); +x_220 = l_Lean_throwErrorAt___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__12(x_7, x_219, x_10, x_11, x_12, x_13, x_14, x_15, x_210); +lean_dec(x_15); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +return x_220; +} +else { -return x_6; +lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; uint8_t x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; uint8_t x_234; +x_221 = lean_ctor_get(x_215, 0); +lean_inc(x_221); +if (lean_is_exclusive(x_215)) { + lean_ctor_release(x_215, 0); + x_222 = x_215; +} else { + lean_dec_ref(x_215); + x_222 = lean_box(0); +} +x_223 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_209, x_10, x_11, x_12, x_13, x_14, x_15, x_210); +x_224 = lean_ctor_get(x_223, 0); +lean_inc(x_224); +x_225 = lean_ctor_get(x_223, 1); +lean_inc(x_225); +if (lean_is_exclusive(x_223)) { + lean_ctor_release(x_223, 0); + lean_ctor_release(x_223, 1); + x_226 = x_223; +} else { + lean_dec_ref(x_223); + x_226 = lean_box(0); +} +lean_inc(x_224); +lean_inc(x_2); +x_227 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_227, 0, x_2); +lean_ctor_set(x_227, 1, x_221); +lean_ctor_set(x_227, 2, x_224); +x_228 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 3); +lean_dec(x_1); +x_229 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_229, 0, x_227); +lean_ctor_set_uint8(x_229, sizeof(void*)*1, x_228); +if (lean_is_scalar(x_222)) { + x_230 = lean_alloc_ctor(0, 1, 0); +} else { + x_230 = x_222; + lean_ctor_set_tag(x_230, 0); +} +lean_ctor_set(x_230, 0, x_229); +x_231 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__7; +x_232 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_231, x_10, x_11, x_12, x_13, x_14, x_15, x_225); +x_233 = lean_ctor_get(x_232, 0); +lean_inc(x_233); +x_234 = lean_unbox(x_233); +lean_dec(x_233); +if (x_234 == 0) +{ +lean_object* x_235; lean_object* x_236; lean_object* x_237; +lean_dec(x_226); +lean_dec(x_224); +lean_dec(x_211); +x_235 = lean_ctor_get(x_232, 1); +lean_inc(x_235); +lean_dec(x_232); +x_236 = lean_box(0); +x_237 = l_Lean_Elab_Command_elabAxiom___lambda__3(x_230, x_2, x_8, x_17, x_236, x_10, x_11, x_12, x_13, x_14, x_15, x_235); +return x_237; } else { -lean_object* x_93; lean_object* x_94; lean_object* x_95; -x_93 = lean_ctor_get(x_6, 0); -x_94 = lean_ctor_get(x_6, 1); -lean_inc(x_94); -lean_inc(x_93); -lean_dec(x_6); -x_95 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_95, 0, x_93); -lean_ctor_set(x_95, 1, x_94); -return x_95; +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; +x_238 = lean_ctor_get(x_232, 1); +lean_inc(x_238); +if (lean_is_exclusive(x_232)) { + lean_ctor_release(x_232, 0); + lean_ctor_release(x_232, 1); + x_239 = x_232; +} else { + lean_dec_ref(x_232); + x_239 = lean_box(0); } +lean_inc(x_2); +x_240 = l_Lean_MessageData_ofName(x_2); +x_241 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__9; +if (lean_is_scalar(x_239)) { + x_242 = lean_alloc_ctor(7, 2, 0); +} else { + x_242 = x_239; + lean_ctor_set_tag(x_242, 7); +} +lean_ctor_set(x_242, 0, x_241); +lean_ctor_set(x_242, 1, x_240); +x_243 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__11; +if (lean_is_scalar(x_226)) { + x_244 = lean_alloc_ctor(7, 2, 0); +} else { + x_244 = x_226; + lean_ctor_set_tag(x_244, 7); +} +lean_ctor_set(x_244, 0, x_242); +lean_ctor_set(x_244, 1, x_243); +x_245 = l_Lean_MessageData_ofExpr(x_224); +if (lean_is_scalar(x_211)) { + x_246 = lean_alloc_ctor(7, 2, 0); +} else { + x_246 = x_211; + lean_ctor_set_tag(x_246, 7); +} +lean_ctor_set(x_246, 0, x_244); +lean_ctor_set(x_246, 1, x_245); +x_247 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_247, 0, x_246); +lean_ctor_set(x_247, 1, x_241); +x_248 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_231, x_247, x_10, x_11, x_12, x_13, x_14, x_15, x_238); +x_249 = lean_ctor_get(x_248, 0); +lean_inc(x_249); +x_250 = lean_ctor_get(x_248, 1); +lean_inc(x_250); +lean_dec(x_248); +x_251 = l_Lean_Elab_Command_elabAxiom___lambda__3(x_230, x_2, x_8, x_17, x_249, x_10, x_11, x_12, x_13, x_14, x_15, x_250); +lean_dec(x_249); +return x_251; } } } -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* 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_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_4); +lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; +lean_dec(x_17); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_5); lean_dec(x_2); lean_dec(x_1); -return x_6; +x_252 = lean_ctor_get(x_204, 0); +lean_inc(x_252); +x_253 = lean_ctor_get(x_204, 1); +lean_inc(x_253); +if (lean_is_exclusive(x_204)) { + lean_ctor_release(x_204, 0); + lean_ctor_release(x_204, 1); + x_254 = x_204; +} else { + lean_dec_ref(x_204); + x_254 = lean_box(0); } +if (lean_is_scalar(x_254)) { + x_255 = lean_alloc_ctor(1, 2, 0); +} else { + x_255 = x_254; } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___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) { -_start: -{ -lean_object* x_6; -x_6 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___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_ctor_set(x_255, 0, x_252); +lean_ctor_set(x_255, 1, x_253); +return x_255; } } -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* 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_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__3(x_1, x_2, x_3, x_4, x_5); +lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; +lean_dec(x_17); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -return x_6; -} +x_256 = lean_ctor_get(x_201, 0); +lean_inc(x_256); +x_257 = lean_ctor_get(x_201, 1); +lean_inc(x_257); +if (lean_is_exclusive(x_201)) { + lean_ctor_release(x_201, 0); + lean_ctor_release(x_201, 1); + x_258 = x_201; +} else { + lean_dec_ref(x_201); + x_258 = lean_box(0); } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -lean_object* x_5; -x_5 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1(x_1, x_2, x_3, x_4); -lean_dec(x_3); -lean_dec(x_1); -return x_5; +if (lean_is_scalar(x_258)) { + x_259 = lean_alloc_ctor(1, 2, 0); +} else { + x_259 = x_258; } +lean_ctor_set(x_259, 0, x_256); +lean_ctor_set(x_259, 1, x_257); +return x_259; } -LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -lean_object* x_7; -x_7 = l_Lean_Elab_addAuxDeclarationRanges___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2(x_1, x_2, x_3, x_4, x_5, x_6); -lean_dec(x_5); -lean_dec(x_3); -lean_dec(x_2); -return x_7; } } -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* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: +else { -lean_object* x_8; -x_8 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +uint8_t x_260; +lean_dec(x_22); +lean_dec(x_17); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_8); lean_dec(x_6); -lean_dec(x_4); -return x_8; -} -} -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* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; -x_9 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_7); lean_dec(x_5); lean_dec(x_4); -return x_9; -} +lean_dec(x_2); +lean_dec(x_1); +x_260 = !lean_is_exclusive(x_28); +if (x_260 == 0) +{ +return x_28; } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: +else { -lean_object* x_9; -x_9 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___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_5); -lean_dec(x_3); -return x_9; +lean_object* x_261; lean_object* x_262; lean_object* x_263; +x_261 = lean_ctor_get(x_28, 0); +x_262 = lean_ctor_get(x_28, 1); +lean_inc(x_262); +lean_inc(x_261); +lean_dec(x_28); +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; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: +} +else { -lean_object* x_8; -x_8 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +uint8_t x_264; +lean_dec(x_22); +lean_dec(x_17); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); +lean_dec(x_2); lean_dec(x_1); -return x_8; -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___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: +x_264 = !lean_is_exclusive(x_26); +if (x_264 == 0) { -size_t x_9; size_t x_10; lean_object* x_11; -x_9 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_10 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_11 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3(x_1, x_2, x_9, x_10, x_5, x_6, x_7, x_8); -lean_dec(x_6); -return x_11; -} +return x_26; } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___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: +else { -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_2); -lean_dec(x_2); -x_9 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__4(x_7, x_8, x_3, x_4, x_5, x_6); -lean_dec(x_5); -lean_dec(x_4); -return x_9; +lean_object* x_265; lean_object* x_266; lean_object* x_267; +x_265 = lean_ctor_get(x_26, 0); +x_266 = lean_ctor_get(x_26, 1); +lean_inc(x_266); +lean_inc(x_265); +lean_dec(x_26); +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_EXPORT lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___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) { -_start: +} +else { -lean_object* x_7; -x_7 = l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6(x_1, x_2, x_3, x_4, x_5, x_6); +uint8_t x_268; +lean_dec(x_17); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_6); lean_dec(x_5); +lean_dec(x_4); lean_dec(x_2); -return x_7; -} +lean_dec(x_1); +x_268 = !lean_is_exclusive(x_21); +if (x_268 == 0) +{ +return x_21; } -LEAN_EXPORT lean_object* l_Lean_Linter_logLintIf___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___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: +else { -lean_object* x_7; -x_7 = l_Lean_Linter_logLintIf___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5(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_269; lean_object* x_270; lean_object* x_271; +x_269 = lean_ctor_get(x_21, 0); +x_270 = lean_ctor_get(x_21, 1); +lean_inc(x_270); +lean_inc(x_269); +lean_dec(x_21); +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_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { -_start: +} +else { -lean_object* x_16; -x_16 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___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); +uint8_t x_272; +lean_dec(x_17); +lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); -return x_16; -} +lean_dec(x_11); +lean_dec(x_10); +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_272 = !lean_is_exclusive(x_19); +if (x_272 == 0) +{ +return x_19; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_classInductiveSyntaxToView(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___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView(x_1, x_2, x_3, x_4, x_5); -return x_6; +lean_object* x_273; lean_object* x_274; lean_object* x_275; +x_273 = lean_ctor_get(x_19, 0); +x_274 = lean_ctor_get(x_19, 1); +lean_inc(x_274); +lean_inc(x_273); +lean_dec(x_19); +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_EXPORT lean_object* l_Lean_Elab_Command_elabInductive(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -lean_object* x_6; -lean_inc(x_4); -lean_inc(x_3); -x_6 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView(x_1, x_2, 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; lean_object* x_11; lean_object* x_12; -x_7 = lean_ctor_get(x_6, 0); +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_14 = l_Lean_Elab_Term_getLevelNames___rarg(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 = lean_ctor_get(x_11, 6); +lean_inc(x_17); +lean_inc(x_11); lean_inc(x_7); -x_8 = lean_ctor_get(x_6, 1); -lean_inc(x_8); -lean_dec(x_6); -x_9 = lean_box(0); -x_10 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_10, 0, x_7); -lean_ctor_set(x_10, 1, x_9); -x_11 = lean_array_mk(x_10); -x_12 = l_Lean_Elab_Command_elabInductiveViews(x_11, x_3, x_4, x_8); -return x_12; +lean_inc(x_2); +lean_inc(x_15); +x_18 = l_Lean_Elab_Term_expandDeclId(x_17, x_15, x_1, x_2, x_7, x_8, x_9, x_10, x_11, x_12, x_16); +if (lean_obj_tag(x_18) == 0) +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +x_20 = lean_ctor_get(x_18, 1); +lean_inc(x_20); +lean_dec(x_18); +x_21 = lean_ctor_get(x_19, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_19, 1); +lean_inc(x_22); +x_23 = lean_ctor_get(x_19, 2); +lean_inc(x_23); +lean_dec(x_19); +x_24 = lean_ctor_get(x_2, 0); +lean_inc(x_24); +lean_inc(x_11); +lean_inc(x_3); +lean_inc(x_22); +x_25 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2(x_22, x_24, x_3, x_7, x_8, x_9, x_10, x_11, x_12, x_20); +x_26 = lean_ctor_get(x_25, 1); +lean_inc(x_26); +lean_dec(x_25); +x_27 = lean_alloc_closure((void*)(l_Lean_Name_beq___boxed), 2, 1); +lean_closure_set(x_27, 0, x_21); +x_28 = l_Lean_Syntax_getArgs(x_4); +lean_inc(x_23); +lean_inc(x_22); +x_29 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabAxiom___lambda__4___boxed), 16, 8); +lean_closure_set(x_29, 0, x_2); +lean_closure_set(x_29, 1, x_22); +lean_closure_set(x_29, 2, x_5); +lean_closure_set(x_29, 3, x_6); +lean_closure_set(x_29, 4, x_15); +lean_closure_set(x_29, 5, x_23); +lean_closure_set(x_29, 6, x_3); +lean_closure_set(x_29, 7, x_1); +x_30 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabBinders___rarg), 9, 2); +lean_closure_set(x_30, 0, x_28); +lean_closure_set(x_30, 1, x_29); +x_31 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withLevelNames___rarg), 9, 2); +lean_closure_set(x_31, 0, x_23); +lean_closure_set(x_31, 1, x_30); +x_32 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withDeclName___rarg), 9, 2); +lean_closure_set(x_32, 0, x_22); +lean_closure_set(x_32, 1, x_31); +x_33 = l_Lean_Elab_Term_withAutoBoundImplicitForbiddenPred___rarg(x_27, x_32, x_7, x_8, x_9, x_10, x_11, x_12, x_26); +return x_33; } else { -uint8_t x_13; -lean_dec(x_4); +uint8_t x_34; +lean_dec(x_15); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); lean_dec(x_3); -x_13 = !lean_is_exclusive(x_6); -if (x_13 == 0) +lean_dec(x_2); +lean_dec(x_1); +x_34 = !lean_is_exclusive(x_18); +if (x_34 == 0) { -return x_6; +return x_18; } else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_14 = lean_ctor_get(x_6, 0); -x_15 = lean_ctor_get(x_6, 1); -lean_inc(x_15); -lean_inc(x_14); -lean_dec(x_6); -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_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_18, 0); +x_36 = lean_ctor_get(x_18, 1); +lean_inc(x_36); +lean_inc(x_35); +lean_dec(x_18); +x_37 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +return x_37; } } } } -static lean_object* _init_l_Lean_Elab_Command_elabClassInductive___closed__1() { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom(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_unchecked("class", 5, 5); -return x_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 = lean_unsigned_to_nat(1u); +x_7 = l_Lean_Syntax_getArg(x_2, x_6); +x_8 = lean_unsigned_to_nat(2u); +x_9 = l_Lean_Syntax_getArg(x_2, x_8); +x_10 = l_Lean_Elab_expandDeclSig(x_9); +lean_dec(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_alloc_closure((void*)(l_Lean_Elab_Command_elabAxiom___lambda__5___boxed), 13, 5); +lean_closure_set(x_13, 0, x_7); +lean_closure_set(x_13, 1, x_1); +lean_closure_set(x_13, 2, x_2); +lean_closure_set(x_13, 3, x_11); +lean_closure_set(x_13, 4, x_12); +x_14 = l_Lean_Elab_Command_runTermElabM___rarg(x_13, x_3, x_4, x_5); +return x_14; } } -static lean_object* _init_l_Lean_Elab_Command_elabClassInductive___closed__2() { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Command_elabClassInductive___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_11; +x_11 = l_Lean_Elab_Command_elabAxiom___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_3); +return x_11; } } -static lean_object* _init_l_Lean_Elab_Command_elabClassInductive___closed__3() { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -uint8_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = 0; -x_2 = l_Lean_Elab_Command_elabClassInductive___closed__2; -x_3 = lean_box(0); -x_4 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_4, 0, x_2); -lean_ctor_set(x_4, 1, x_3); -lean_ctor_set_uint8(x_4, sizeof(void*)*2, x_1); -return x_4; +lean_object* x_13; +x_13 = 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, x_11, x_12); +lean_dec(x_5); +return x_13; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabClassInductive(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { -lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_6 = l_Lean_Elab_Command_elabClassInductive___closed__3; -x_7 = l_Lean_Elab_Modifiers_addAttr(x_1, x_6); -lean_inc(x_4); -lean_inc(x_3); -x_8 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView(x_7, x_2, x_3, x_4, x_5); -if (lean_obj_tag(x_8) == 0) +lean_object* x_17; +x_17 = l_Lean_Elab_Command_elabAxiom___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +lean_dec(x_9); +lean_dec(x_7); +return x_17; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___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) { +_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_8, 0); -lean_inc(x_9); -x_10 = lean_ctor_get(x_8, 1); -lean_inc(x_10); -lean_dec(x_8); -x_11 = lean_box(0); -x_12 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_12, 0, x_9); -lean_ctor_set(x_12, 1, x_11); -x_13 = lean_array_mk(x_12); -x_14 = l_Lean_Elab_Command_elabInductiveViews(x_13, x_3, x_4, x_10); +lean_object* x_14; +x_14 = l_Lean_Elab_Command_elabAxiom___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); +lean_dec(x_4); return x_14; } -else +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___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_15; +lean_object* x_6; +x_6 = l_Lean_Elab_Command_elabAxiom(x_1, x_2, x_3, x_4, x_5); lean_dec(x_4); lean_dec(x_3); -x_15 = !lean_is_exclusive(x_8); -if (x_15 == 0) -{ -return x_8; -} -else -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_8, 0); -x_17 = lean_ctor_get(x_8, 1); -lean_inc(x_17); -lean_inc(x_16); -lean_dec(x_8); -x_18 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_18, 0, x_16); -lean_ctor_set(x_18, 1, x_17); -return x_18; -} -} +return x_6; } } static lean_object* _init_l_Lean_Elab_Command_expandNamespacedDeclaration___closed__1() { @@ -6413,6 +3922,7 @@ x_8 = lean_ctor_get(x_6, 1); lean_inc(x_8); lean_dec(x_6); x_9 = l_Lean_Elab_Command_elabAxiom(x_7, x_2, x_3, x_4, x_8); +lean_dec(x_3); return x_9; } else @@ -6480,43 +3990,43 @@ lean_inc(x_6); x_8 = l_Lean_Elab_Command_isDefLike(x_6); if (x_8 == 0) { -lean_object* x_9; uint8_t x_10; -x_9 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__15; -x_10 = lean_name_eq(x_7, x_9); -if (x_10 == 0) -{ -lean_object* x_11; uint8_t x_12; -x_11 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__17; +lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; +x_9 = lean_unsigned_to_nat(0u); +x_10 = l_Lean_Syntax_getArg(x_1, x_9); +lean_dec(x_1); +x_11 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__15; x_12 = lean_name_eq(x_7, x_11); if (x_12 == 0) { lean_object* x_13; uint8_t x_14; -x_13 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__19; +x_13 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__17; x_14 = lean_name_eq(x_7, x_13); if (x_14 == 0) { lean_object* x_15; uint8_t x_16; -x_15 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__21; +x_15 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__19; x_16 = lean_name_eq(x_7, x_15); -lean_dec(x_7); if (x_16 == 0) { -uint8_t x_17; lean_object* x_18; lean_object* x_19; +lean_object* x_17; uint8_t x_18; +x_17 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__21; +x_18 = lean_name_eq(x_7, x_17); +lean_dec(x_7); +if (x_18 == 0) +{ +uint8_t x_19; lean_object* x_20; lean_object* x_21; +lean_dec(x_10); lean_dec(x_6); -lean_dec(x_1); -x_17 = 1; -x_18 = l_Lean_Elab_Command_elabDeclaration___closed__3; -x_19 = l_Lean_Elab_Command_withoutCommandIncrementality___rarg(x_17, x_18, x_2, x_3, x_4); -return x_19; +x_19 = 1; +x_20 = l_Lean_Elab_Command_elabDeclaration___closed__3; +x_21 = l_Lean_Elab_Command_withoutCommandIncrementality___rarg(x_19, x_20, x_2, x_3, x_4); +return x_21; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; lean_object* x_24; -x_20 = lean_unsigned_to_nat(0u); -x_21 = l_Lean_Syntax_getArg(x_1, x_20); -lean_dec(x_1); -x_22 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabDeclaration___lambda__1___boxed), 5, 2); -lean_closure_set(x_22, 0, x_21); +lean_object* x_22; uint8_t x_23; lean_object* x_24; +x_22 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabDeclaration___lambda__1), 5, 2); +lean_closure_set(x_22, 0, x_10); lean_closure_set(x_22, 1, x_6); x_23 = 1; x_24 = l_Lean_Elab_Command_withoutCommandIncrementality___rarg(x_23, x_22, x_2, x_3, x_4); @@ -6525,89 +4035,53 @@ return x_24; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; lean_object* x_29; +lean_object* x_25; uint8_t x_26; lean_object* x_27; lean_dec(x_7); -x_25 = lean_unsigned_to_nat(0u); -x_26 = l_Lean_Syntax_getArg(x_1, x_25); -lean_dec(x_1); -x_27 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabDeclaration___lambda__2___boxed), 5, 2); -lean_closure_set(x_27, 0, x_26); -lean_closure_set(x_27, 1, x_6); -x_28 = 1; -x_29 = l_Lean_Elab_Command_withoutCommandIncrementality___rarg(x_28, x_27, x_2, x_3, x_4); -return x_29; -} -} -else -{ -lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; lean_object* x_34; -lean_dec(x_7); -x_30 = lean_unsigned_to_nat(0u); -x_31 = l_Lean_Syntax_getArg(x_1, x_30); -lean_dec(x_1); -x_32 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabDeclaration___lambda__3___boxed), 5, 2); -lean_closure_set(x_32, 0, x_31); -lean_closure_set(x_32, 1, x_6); -x_33 = 1; -x_34 = l_Lean_Elab_Command_withoutCommandIncrementality___rarg(x_33, x_32, x_2, x_3, x_4); -return x_34; -} -} -else -{ -lean_object* x_35; lean_object* x_36; lean_object* x_37; uint8_t x_38; lean_object* x_39; -lean_dec(x_7); -x_35 = lean_unsigned_to_nat(0u); -x_36 = l_Lean_Syntax_getArg(x_1, x_35); -lean_dec(x_1); -x_37 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabDeclaration___lambda__4___boxed), 5, 2); -lean_closure_set(x_37, 0, x_36); -lean_closure_set(x_37, 1, x_6); -x_38 = 1; -x_39 = l_Lean_Elab_Command_withoutCommandIncrementality___rarg(x_38, x_37, x_2, x_3, x_4); -return x_39; -} -} -else -{ -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; -lean_dec(x_7); -lean_dec(x_6); -x_40 = lean_box(0); -x_41 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_41, 0, x_1); -lean_ctor_set(x_41, 1, x_40); -x_42 = lean_array_mk(x_41); -x_43 = l_Lean_Elab_Command_elabMutualDef(x_42, x_2, x_3, x_4); -return x_43; -} +x_25 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabDeclaration___lambda__2), 5, 2); +lean_closure_set(x_25, 0, x_10); +lean_closure_set(x_25, 1, x_6); +x_26 = 1; +x_27 = l_Lean_Elab_Command_withoutCommandIncrementality___rarg(x_26, x_25, x_2, x_3, x_4); +return x_27; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabDeclaration___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: +else { -lean_object* x_6; -x_6 = l_Lean_Elab_Command_elabDeclaration___lambda__1(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_1); -return x_6; +lean_object* x_28; uint8_t x_29; lean_object* x_30; +lean_dec(x_7); +x_28 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabDeclaration___lambda__3), 5, 2); +lean_closure_set(x_28, 0, x_10); +lean_closure_set(x_28, 1, x_6); +x_29 = 1; +x_30 = l_Lean_Elab_Command_withoutCommandIncrementality___rarg(x_29, x_28, x_2, x_3, x_4); +return x_30; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabDeclaration___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: +else { -lean_object* x_6; -x_6 = l_Lean_Elab_Command_elabDeclaration___lambda__2(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_1); -return x_6; +lean_object* x_31; uint8_t x_32; lean_object* x_33; +lean_dec(x_7); +x_31 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabDeclaration___lambda__4___boxed), 5, 2); +lean_closure_set(x_31, 0, x_10); +lean_closure_set(x_31, 1, x_6); +x_32 = 1; +x_33 = l_Lean_Elab_Command_withoutCommandIncrementality___rarg(x_32, x_31, x_2, x_3, x_4); +return x_33; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabDeclaration___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: +else { -lean_object* x_6; -x_6 = l_Lean_Elab_Command_elabDeclaration___lambda__3(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_1); -return x_6; +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; +lean_dec(x_7); +lean_dec(x_6); +x_34 = lean_box(0); +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_1); +lean_ctor_set(x_35, 1, x_34); +x_36 = lean_array_mk(x_35); +x_37 = l_Lean_Elab_Command_elabMutualDef(x_36, x_2, x_3, x_4); +return x_37; +} } } LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabDeclaration___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { @@ -6616,7 +4090,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabDeclaration___lambda__4___boxed lean_object* x_6; x_6 = l_Lean_Elab_Command_elabDeclaration___lambda__4(x_1, x_2, x_3, x_4, x_5); lean_dec(x_4); -lean_dec(x_1); return x_6; } } @@ -6772,284 +4245,11 @@ return x_4; } LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclaration__2(lean_object* x_1) { _start: -{ -lean_object* x_2; lean_object* x_3; -x_2 = l___regBuiltin_Lean_Elab_Command_elabDeclaration__1___closed__2; -x_3 = l_Lean_Elab_addBuiltinIncrementalElab(x_2, x_1); -return x_3; -} -} -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualInductive___spec__1(lean_object* x_1, size_t x_2, size_t x_3) { -_start: -{ -uint8_t x_4; -x_4 = lean_usize_dec_eq(x_2, x_3); -if (x_4 == 0) -{ -lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; -x_5 = lean_array_uget(x_1, x_2); -x_6 = lean_unsigned_to_nat(1u); -x_7 = l_Lean_Syntax_getArg(x_5, x_6); -lean_dec(x_5); -x_8 = l_Lean_Syntax_getKind(x_7); -x_9 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__17; -x_10 = lean_name_eq(x_8, x_9); -lean_dec(x_8); -if (x_10 == 0) -{ -uint8_t x_11; -x_11 = 1; -return x_11; -} -else -{ -size_t x_12; size_t x_13; -x_12 = 1; -x_13 = lean_usize_add(x_2, x_12); -x_2 = x_13; -goto _start; -} -} -else -{ -uint8_t x_15; -x_15 = 0; -return x_15; -} -} -} -LEAN_EXPORT uint8_t l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualInductive(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; uint8_t x_7; -x_2 = lean_unsigned_to_nat(1u); -x_3 = l_Lean_Syntax_getArg(x_1, x_2); -x_4 = l_Lean_Syntax_getArgs(x_3); -lean_dec(x_3); -x_5 = lean_array_get_size(x_4); -x_6 = lean_unsigned_to_nat(0u); -x_7 = lean_nat_dec_lt(x_6, x_5); -if (x_7 == 0) -{ -uint8_t x_8; -lean_dec(x_5); -lean_dec(x_4); -x_8 = 1; -return x_8; -} -else -{ -size_t x_9; size_t x_10; uint8_t x_11; -x_9 = 0; -x_10 = lean_usize_of_nat(x_5); -lean_dec(x_5); -x_11 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualInductive___spec__1(x_4, x_9, x_10); -lean_dec(x_4); -if (x_11 == 0) -{ -uint8_t x_12; -x_12 = 1; -return x_12; -} -else -{ -uint8_t x_13; -x_13 = 0; -return x_13; -} -} -} -} -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualInductive___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -size_t x_4; size_t x_5; uint8_t x_6; lean_object* x_7; -x_4 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_5 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_6 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualInductive___spec__1(x_1, x_4, x_5); -lean_dec(x_1); -x_7 = lean_box(x_6); -return x_7; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualInductive___boxed(lean_object* x_1) { -_start: -{ -uint8_t x_2; lean_object* x_3; -x_2 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualInductive(x_1); -lean_dec(x_1); -x_3 = lean_box(x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_elabMutualInductive___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) { -_start: -{ -uint8_t x_7; -x_7 = lean_usize_dec_lt(x_2, x_1); -if (x_7 == 0) -{ -lean_object* x_8; -lean_dec(x_5); -lean_dec(x_4); -x_8 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_8, 0, x_3); -lean_ctor_set(x_8, 1, x_6); -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_3, x_2); -x_10 = lean_unsigned_to_nat(0u); -x_11 = lean_array_uset(x_3, x_2, x_10); -x_12 = l_Lean_Syntax_getArg(x_9, x_10); -lean_inc(x_4); -x_13 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1(x_12, x_4, x_5, x_6); -lean_dec(x_12); -if (lean_obj_tag(x_13) == 0) -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; -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_unsigned_to_nat(1u); -x_17 = l_Lean_Syntax_getArg(x_9, x_16); -lean_dec(x_9); -lean_inc(x_5); -lean_inc(x_4); -x_18 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView(x_14, x_17, x_4, x_5, x_15); -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_11, x_2, x_19); -x_2 = x_22; -x_3 = x_23; -x_6 = x_20; -goto _start; -} -else -{ -uint8_t x_25; -lean_dec(x_11); -lean_dec(x_5); -lean_dec(x_4); -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; -} -} -} -else -{ -uint8_t x_29; -lean_dec(x_11); -lean_dec(x_9); -lean_dec(x_5); -lean_dec(x_4); -x_29 = !lean_is_exclusive(x_13); -if (x_29 == 0) -{ -return x_13; -} -else -{ -lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_30 = lean_ctor_get(x_13, 0); -x_31 = lean_ctor_get(x_13, 1); -lean_inc(x_31); -lean_inc(x_30); -lean_dec(x_13); -x_32 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_32, 0, x_30); -lean_ctor_set(x_32, 1, x_31); -return x_32; -} -} -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_elabMutualInductive(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_array_size(x_1); -x_6 = 0; -lean_inc(x_3); -lean_inc(x_2); -x_7 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_elabMutualInductive___spec__1(x_5, x_6, x_1, 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; -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_Elab_Command_elabInductiveViews(x_8, x_2, x_3, x_9); -return x_10; -} -else -{ -uint8_t x_11; -lean_dec(x_3); -lean_dec(x_2); -x_11 = !lean_is_exclusive(x_7); -if (x_11 == 0) -{ -return x_7; -} -else -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_12 = lean_ctor_get(x_7, 0); -x_13 = lean_ctor_get(x_7, 1); -lean_inc(x_13); -lean_inc(x_12); -lean_dec(x_7); -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_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_elabMutualInductive___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -size_t x_7; size_t x_8; lean_object* x_9; -x_7 = lean_unbox_usize(x_1); -lean_dec(x_1); -x_8 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_9 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_elabMutualInductive___spec__1(x_7, x_8, x_3, x_4, x_5, x_6); -return x_9; +{ +lean_object* x_2; lean_object* x_3; +x_2 = l___regBuiltin_Lean_Elab_Command_elabDeclaration__1___closed__2; +x_3 = l_Lean_Elab_addBuiltinIncrementalElab(x_2, x_1); +return x_3; } } LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualDef___spec__1(lean_object* x_1, size_t x_2, size_t x_3) { @@ -7673,7 +4873,7 @@ static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Elab_Command_expandMu lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_setDeclIdName___closed__5; x_2 = l_Array_mapMUnsafe_map___at_Lean_Elab_Command_expandMutualNamespace___spec__3___closed__1; -x_3 = lean_unsigned_to_nat(308u); +x_3 = lean_unsigned_to_nat(241u); x_4 = lean_unsigned_to_nat(40u); x_5 = l_Array_mapMUnsafe_map___at_Lean_Elab_Command_expandMutualNamespace___spec__3___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -9302,7 +6502,7 @@ x_5 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualDef(x_1); if (x_5 == 0) { uint8_t x_6; -x_6 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualInductive(x_1); +x_6 = l_Lean_Elab_Command_isMutualInductive(x_1); if (x_6 == 0) { uint8_t x_7; lean_object* x_8; lean_object* x_9; @@ -9318,7 +6518,7 @@ x_10 = lean_unsigned_to_nat(1u); x_11 = l_Lean_Syntax_getArg(x_1, x_10); x_12 = l_Lean_Syntax_getArgs(x_11); lean_dec(x_11); -x_13 = lean_alloc_closure((void*)(l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_elabMutualInductive), 4, 1); +x_13 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabMutualInductive), 4, 1); lean_closure_set(x_13, 0, x_12); x_14 = 1; x_15 = l_Lean_Elab_Command_withoutCommandIncrementality___rarg(x_14, x_13, x_2, x_3, x_4); @@ -9702,1288 +6902,1863 @@ goto _start; } } } -else +else +{ +lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; uint8_t x_68; +x_64 = lean_ctor_get(x_4, 0); +x_65 = lean_ctor_get(x_4, 1); +lean_inc(x_65); +lean_inc(x_64); +lean_dec(x_4); +lean_inc(x_10); +x_66 = l_Lean_Syntax_getKind(x_10); +x_67 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__2; +x_68 = lean_name_eq(x_66, x_67); +lean_dec(x_66); +if (x_68 == 0) +{ +lean_object* x_69; lean_object* x_70; size_t x_71; size_t x_72; +x_69 = lean_array_push(x_64, x_10); +x_70 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_70, 0, x_69); +lean_ctor_set(x_70, 1, x_65); +x_71 = 1; +x_72 = lean_usize_add(x_3, x_71); +x_3 = x_72; +x_4 = x_70; +goto _start; +} +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; uint8_t x_83; +x_74 = lean_unsigned_to_nat(1u); +x_75 = l_Lean_Syntax_getArg(x_10, x_74); +x_76 = l_Lean_Syntax_getId(x_75); +lean_dec(x_75); +x_77 = lean_erase_macro_scopes(x_76); +x_78 = lean_st_ref_get(x_6, x_7); +x_79 = lean_ctor_get(x_78, 0); +lean_inc(x_79); +x_80 = lean_ctor_get(x_78, 1); +lean_inc(x_80); +if (lean_is_exclusive(x_78)) { + lean_ctor_release(x_78, 0); + lean_ctor_release(x_78, 1); + x_81 = x_78; +} else { + lean_dec_ref(x_78); + x_81 = lean_box(0); +} +x_82 = lean_ctor_get(x_79, 0); +lean_inc(x_82); +lean_dec(x_79); +x_83 = l_Lean_isAttribute(x_82, x_77); +lean_dec(x_82); +if (x_83 == 0) +{ +lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; uint8_t x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; size_t x_93; size_t x_94; +x_84 = l_Lean_MessageData_ofName(x_77); +x_85 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__4; +if (lean_is_scalar(x_81)) { + x_86 = lean_alloc_ctor(7, 2, 0); +} else { + x_86 = x_81; + lean_ctor_set_tag(x_86, 7); +} +lean_ctor_set(x_86, 0, x_85); +lean_ctor_set(x_86, 1, x_84); +x_87 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__6; +x_88 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_88, 0, x_86); +lean_ctor_set(x_88, 1, x_87); +x_89 = 2; +lean_inc(x_5); +x_90 = l_Lean_logAt___at_Lean_Elab_Command_runLinters___spec__2(x_10, x_88, x_89, x_5, x_6, x_80); +lean_dec(x_10); +x_91 = lean_ctor_get(x_90, 1); +lean_inc(x_91); +lean_dec(x_90); +x_92 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_92, 0, x_64); +lean_ctor_set(x_92, 1, x_65); +x_93 = 1; +x_94 = lean_usize_add(x_3, x_93); +x_3 = x_94; +x_4 = x_92; +x_7 = x_91; +goto _start; +} +else +{ +lean_object* x_96; lean_object* x_97; size_t x_98; size_t x_99; +lean_dec(x_81); +lean_dec(x_10); +x_96 = lean_array_push(x_65, x_77); +x_97 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_97, 0, x_64); +lean_ctor_set(x_97, 1, x_96); +x_98 = 1; +x_99 = lean_usize_add(x_3, x_98); +x_3 = x_99; +x_4 = x_97; +x_7 = x_80; +goto _start; +} +} +} +} +} +} +static lean_object* _init_l_panic___at_Lean_Elab_Command_elabAttr___spec__3___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Term_instMonadTermElabM; +x_2 = l_Lean_instInhabitedName; +x_3 = l_instInhabitedOfMonad___rarg(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_Command_elabAttr___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; lean_object* x_10; lean_object* x_11; +x_9 = l_panic___at_Lean_Elab_Command_elabAttr___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; +} +} +static lean_object* _init_l_Lean_ensureNonAmbiguous___at_Lean_Elab_Command_elabAttr___spec__2___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean.ResolveName", 16, 16); +return x_1; +} +} +static lean_object* _init_l_Lean_ensureNonAmbiguous___at_Lean_Elab_Command_elabAttr___spec__2___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean.ensureNonAmbiguous", 23, 23); +return x_1; +} +} +static lean_object* _init_l_Lean_ensureNonAmbiguous___at_Lean_Elab_Command_elabAttr___spec__2___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l_Lean_ensureNonAmbiguous___at_Lean_Elab_Command_elabAttr___spec__2___closed__1; +x_2 = l_Lean_ensureNonAmbiguous___at_Lean_Elab_Command_elabAttr___spec__2___closed__2; +x_3 = lean_unsigned_to_nat(364u); +x_4 = lean_unsigned_to_nat(11u); +x_5 = l_Array_mapMUnsafe_map___at_Lean_Elab_Command_expandMutualNamespace___spec__3___closed__2; +x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +static lean_object* _init_l_Lean_ensureNonAmbiguous___at_Lean_Elab_Command_elabAttr___spec__2___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("ambiguous identifier '", 22, 22); +return x_1; +} +} +static lean_object* _init_l_Lean_ensureNonAmbiguous___at_Lean_Elab_Command_elabAttr___spec__2___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("', possible interpretations: ", 29, 29); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_ensureNonAmbiguous___at_Lean_Elab_Command_elabAttr___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_10; lean_object* x_11; +lean_dec(x_1); +x_10 = l_Lean_ensureNonAmbiguous___at_Lean_Elab_Command_elabAttr___spec__2___closed__3; +x_11 = l_panic___at_Lean_Elab_Command_elabAttr___spec__3(x_10, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_11; +} +else +{ +lean_object* x_12; +x_12 = lean_ctor_get(x_2, 1); +lean_inc(x_12); +if (lean_obj_tag(x_12) == 0) +{ +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_2); +if (x_13 == 0) +{ +lean_object* x_14; +x_14 = lean_ctor_get(x_2, 1); +lean_dec(x_14); +lean_ctor_set_tag(x_2, 0); +lean_ctor_set(x_2, 1, x_9); +return x_2; +} +else +{ +lean_object* x_15; lean_object* x_16; +x_15 = lean_ctor_get(x_2, 0); +lean_inc(x_15); +lean_dec(x_2); +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_16, 1, x_9); +return x_16; +} +} +else +{ +lean_object* x_17; uint8_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; +lean_dec(x_12); +x_17 = lean_box(0); +x_18 = 0; +x_19 = lean_unsigned_to_nat(0u); +lean_inc(x_1); +x_20 = l_Lean_Syntax_formatStxAux(x_17, x_18, x_19, x_1); +x_21 = l_Std_Format_defWidth; +x_22 = lean_format_pretty(x_20, x_21, x_19, x_19); +x_23 = l_Lean_ensureNonAmbiguous___at_Lean_Elab_Command_elabAttr___spec__2___closed__4; +x_24 = lean_string_append(x_23, x_22); +lean_dec(x_22); +x_25 = l_Lean_ensureNonAmbiguous___at_Lean_Elab_Command_elabAttr___spec__2___closed__5; +x_26 = lean_string_append(x_24, x_25); +x_27 = lean_box(0); +x_28 = l_List_mapTR_loop___at_Lean_ensureNonAmbiguous___spec__2(x_2, x_27); +x_29 = l_List_toString___at_Lean_ensureNoOverload___spec__2(x_28); +lean_dec(x_28); +x_30 = lean_string_append(x_26, x_29); +lean_dec(x_29); +x_31 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__8; +x_32 = lean_string_append(x_30, x_31); +x_33 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_33, 0, x_32); +x_34 = l_Lean_MessageData_ofFormat(x_33); +x_35 = l_Lean_throwErrorAt___at_Lean_Elab_Term_processDefDeriving___spec__2(x_1, x_34, 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_1); +return x_35; +} +} +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__4(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_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; uint8_t x_68; -x_64 = lean_ctor_get(x_4, 0); -x_65 = lean_ctor_get(x_4, 1); -lean_inc(x_65); -lean_inc(x_64); -lean_dec(x_4); -lean_inc(x_10); -x_66 = l_Lean_Syntax_getKind(x_10); -x_67 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__2; -x_68 = lean_name_eq(x_66, x_67); -lean_dec(x_66); -if (x_68 == 0) +uint8_t x_13; +x_13 = lean_usize_dec_lt(x_4, x_3); +if (x_13 == 0) { -lean_object* x_69; lean_object* x_70; size_t x_71; size_t x_72; -x_69 = lean_array_push(x_64, x_10); -x_70 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_70, 0, x_69); -lean_ctor_set(x_70, 1, x_65); -x_71 = 1; -x_72 = lean_usize_add(x_3, x_71); -x_3 = x_72; -x_4 = x_70; -goto _start; +lean_object* x_14; +lean_dec(x_11); +lean_dec(x_10); +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_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; uint8_t x_83; -x_74 = lean_unsigned_to_nat(1u); -x_75 = l_Lean_Syntax_getArg(x_10, x_74); -x_76 = l_Lean_Syntax_getId(x_75); -lean_dec(x_75); -x_77 = lean_erase_macro_scopes(x_76); -x_78 = lean_st_ref_get(x_6, x_7); -x_79 = lean_ctor_get(x_78, 0); -lean_inc(x_79); -x_80 = lean_ctor_get(x_78, 1); -lean_inc(x_80); -if (lean_is_exclusive(x_78)) { - lean_ctor_release(x_78, 0); - lean_ctor_release(x_78, 1); - x_81 = x_78; -} else { - lean_dec_ref(x_78); - x_81 = lean_box(0); -} -x_82 = lean_ctor_get(x_79, 0); -lean_inc(x_82); -lean_dec(x_79); -x_83 = l_Lean_isAttribute(x_82, x_77); -lean_dec(x_82); -if (x_83 == 0) +lean_object* x_15; lean_object* x_16; +lean_dec(x_5); +x_15 = lean_array_uget(x_2, x_4); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_1); +x_16 = l_Lean_Attribute_erase(x_1, x_15, x_10, x_11, x_12); +if (lean_obj_tag(x_16) == 0) { -lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; uint8_t x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; size_t x_93; size_t x_94; -x_84 = l_Lean_MessageData_ofName(x_77); -x_85 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__4; -if (lean_is_scalar(x_81)) { - x_86 = lean_alloc_ctor(7, 2, 0); -} else { - x_86 = x_81; - lean_ctor_set_tag(x_86, 7); -} -lean_ctor_set(x_86, 0, x_85); -lean_ctor_set(x_86, 1, x_84); -x_87 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__6; -x_88 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_88, 0, x_86); -lean_ctor_set(x_88, 1, x_87); -x_89 = 2; -lean_inc(x_5); -x_90 = l_Lean_logAt___at_Lean_Elab_Command_runLinters___spec__2(x_10, x_88, x_89, x_5, x_6, x_80); -lean_dec(x_10); -x_91 = lean_ctor_get(x_90, 1); -lean_inc(x_91); -lean_dec(x_90); -x_92 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_92, 0, x_64); -lean_ctor_set(x_92, 1, x_65); -x_93 = 1; -x_94 = lean_usize_add(x_3, x_93); -x_3 = x_94; -x_4 = x_92; -x_7 = x_91; +lean_object* x_17; size_t x_18; size_t x_19; lean_object* x_20; +x_17 = lean_ctor_get(x_16, 1); +lean_inc(x_17); +lean_dec(x_16); +x_18 = 1; +x_19 = lean_usize_add(x_4, x_18); +x_20 = lean_box(0); +x_4 = x_19; +x_5 = x_20; +x_12 = x_17; goto _start; } else { -lean_object* x_96; lean_object* x_97; size_t x_98; size_t x_99; -lean_dec(x_81); +uint8_t x_22; +lean_dec(x_11); lean_dec(x_10); -x_96 = lean_array_push(x_65, x_77); -x_97 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_97, 0, x_64); -lean_ctor_set(x_97, 1, x_96); -x_98 = 1; -x_99 = lean_usize_add(x_3, x_98); -x_3 = x_99; -x_4 = x_97; -x_7 = x_80; -goto _start; +lean_dec(x_1); +x_22 = !lean_is_exclusive(x_16); +if (x_22 == 0) +{ +return x_16; } +else +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_16, 0); +x_24 = lean_ctor_get(x_16, 1); +lean_inc(x_24); +lean_inc(x_23); +lean_dec(x_16); +x_25 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +return x_25; } } } } } -static lean_object* _init_l_panic___at_Lean_Elab_Command_elabAttr___spec__3___closed__1() { +static lean_object* _init_l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabAttr___spec__5___closed__1() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_instMonadTermElabM; -x_2 = l_Lean_instInhabitedName; -x_3 = l_instInhabitedOfMonad___rarg(x_1, x_2); -return x_3; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("unknown constant '", 18, 18); +return x_1; } } -LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_Command_elabAttr___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_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabAttr___spec__5___closed__2() { _start: { -lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_9 = l_panic___at_Lean_Elab_Command_elabAttr___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; lean_object* x_2; +x_1 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabAttr___spec__5___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -static lean_object* _init_l_Lean_ensureNonAmbiguous___at_Lean_Elab_Command_elabAttr___spec__2___closed__1() { +static lean_object* _init_l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabAttr___spec__5___closed__3() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("Lean.ResolveName", 16, 16); +x_1 = lean_mk_string_unchecked("'", 1, 1); return x_1; } } -static lean_object* _init_l_Lean_ensureNonAmbiguous___at_Lean_Elab_Command_elabAttr___spec__2___closed__2() { +static lean_object* _init_l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabAttr___spec__5___closed__4() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Lean.ensureNonAmbiguous", 23, 23); -return x_1; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabAttr___spec__5___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -static lean_object* _init_l_Lean_ensureNonAmbiguous___at_Lean_Elab_Command_elabAttr___spec__2___closed__3() { +LEAN_EXPORT lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabAttr___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_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_ensureNonAmbiguous___at_Lean_Elab_Command_elabAttr___spec__2___closed__1; -x_2 = l_Lean_ensureNonAmbiguous___at_Lean_Elab_Command_elabAttr___spec__2___closed__2; -x_3 = lean_unsigned_to_nat(364u); -x_4 = lean_unsigned_to_nat(11u); -x_5 = l_Array_mapMUnsafe_map___at_Lean_Elab_Command_expandMutualNamespace___spec__3___closed__2; -x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); -return x_6; +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_9 = lean_box(0); +x_10 = l_Lean_Expr_const___override(x_1, x_9); +x_11 = l_Lean_MessageData_ofExpr(x_10); +x_12 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabAttr___spec__5___closed__2; +x_13 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_11); +x_14 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabAttr___spec__5___closed__4; +x_15 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_15, 0, x_13); +lean_ctor_set(x_15, 1, x_14); +x_16 = l_Lean_throwError___at_Lean_Elab_Term_expandDeclId___spec__11(x_15, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +return x_16; } } -static lean_object* _init_l_Lean_ensureNonAmbiguous___at_Lean_Elab_Command_elabAttr___spec__2___closed__4() { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__6___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, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("ambiguous identifier '", 22, 22); -return x_1; -} +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); +x_13 = l_Lean_ensureNonAmbiguous___at_Lean_Elab_Command_elabAttr___spec__2(x_1, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_13) == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_13, 1); +lean_inc(x_15); +lean_dec(x_13); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_14); +x_16 = l_Lean_Elab_Term_applyAttributes(x_14, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_15); +if (lean_obj_tag(x_16) == 0) +{ +lean_object* x_17; size_t 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 = lean_array_size(x_3); +x_19 = lean_box(0); +x_20 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__4(x_14, x_3, x_18, x_4, x_19, x_6, x_7, x_8, x_9, x_10, x_11, x_17); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +if (lean_obj_tag(x_20) == 0) +{ +uint8_t x_21; +x_21 = !lean_is_exclusive(x_20); +if (x_21 == 0) +{ +lean_object* x_22; +x_22 = lean_ctor_get(x_20, 0); +lean_dec(x_22); +lean_ctor_set(x_20, 0, x_19); +return x_20; } -static lean_object* _init_l_Lean_ensureNonAmbiguous___at_Lean_Elab_Command_elabAttr___spec__2___closed__5() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("', possible interpretations: ", 29, 29); -return x_1; +lean_object* x_23; lean_object* x_24; +x_23 = lean_ctor_get(x_20, 1); +lean_inc(x_23); +lean_dec(x_20); +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_19); +lean_ctor_set(x_24, 1, x_23); +return x_24; } } -LEAN_EXPORT lean_object* l_Lean_ensureNonAmbiguous___at_Lean_Elab_Command_elabAttr___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +else { -if (lean_obj_tag(x_2) == 0) +uint8_t x_25; +x_25 = !lean_is_exclusive(x_20); +if (x_25 == 0) { -lean_object* x_10; lean_object* x_11; -lean_dec(x_1); -x_10 = l_Lean_ensureNonAmbiguous___at_Lean_Elab_Command_elabAttr___spec__2___closed__3; -x_11 = l_panic___at_Lean_Elab_Command_elabAttr___spec__3(x_10, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_11; +return x_20; } else { -lean_object* x_12; -x_12 = lean_ctor_get(x_2, 1); -lean_inc(x_12); -if (lean_obj_tag(x_12) == 0) +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_20, 0); +x_27 = lean_ctor_get(x_20, 1); +lean_inc(x_27); +lean_inc(x_26); +lean_dec(x_20); +x_28 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +return x_28; +} +} +} +else { -uint8_t x_13; +uint8_t x_29; +lean_dec(x_14); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_13 = !lean_is_exclusive(x_2); -if (x_13 == 0) +x_29 = !lean_is_exclusive(x_16); +if (x_29 == 0) { -lean_object* x_14; -x_14 = lean_ctor_get(x_2, 1); -lean_dec(x_14); -lean_ctor_set_tag(x_2, 0); -lean_ctor_set(x_2, 1, x_9); -return x_2; +return x_16; } else { -lean_object* x_15; lean_object* x_16; -x_15 = lean_ctor_get(x_2, 0); -lean_inc(x_15); -lean_dec(x_2); -x_16 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_16, 0, x_15); -lean_ctor_set(x_16, 1, x_9); -return x_16; +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_16, 0); +x_31 = lean_ctor_get(x_16, 1); +lean_inc(x_31); +lean_inc(x_30); +lean_dec(x_16); +x_32 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_31); +return x_32; +} } } else { -lean_object* x_17; uint8_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; -lean_dec(x_12); -x_17 = lean_box(0); -x_18 = 0; -x_19 = lean_unsigned_to_nat(0u); -lean_inc(x_1); -x_20 = l_Lean_Syntax_formatStxAux(x_17, x_18, x_19, x_1); -x_21 = l_Std_Format_defWidth; -x_22 = lean_format_pretty(x_20, x_21, x_19, x_19); -x_23 = l_Lean_ensureNonAmbiguous___at_Lean_Elab_Command_elabAttr___spec__2___closed__4; -x_24 = lean_string_append(x_23, x_22); -lean_dec(x_22); -x_25 = l_Lean_ensureNonAmbiguous___at_Lean_Elab_Command_elabAttr___spec__2___closed__5; -x_26 = lean_string_append(x_24, x_25); -x_27 = lean_box(0); -x_28 = l_List_mapTR_loop___at_Lean_ensureNonAmbiguous___spec__2(x_2, x_27); -x_29 = l_List_toString___at_Lean_ensureNoOverload___spec__2(x_28); -lean_dec(x_28); -x_30 = lean_string_append(x_26, x_29); -lean_dec(x_29); -x_31 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__8; -x_32 = lean_string_append(x_30, x_31); -x_33 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_33, 0, x_32); -x_34 = l_Lean_MessageData_ofFormat(x_33); -x_35 = l_Lean_throwErrorAt___at_Lean_Elab_Term_processDefDeriving___spec__2(x_1, x_34, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +uint8_t x_33; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_1); -return x_35; +lean_dec(x_2); +x_33 = !lean_is_exclusive(x_13); +if (x_33 == 0) +{ +return x_13; } +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_13, 0); +x_35 = lean_ctor_get(x_13, 1); +lean_inc(x_35); +lean_inc(x_34); +lean_dec(x_13); +x_36 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_36, 0, x_34); +lean_ctor_set(x_36, 1, x_35); +return x_36; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__4(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_Command_elabAttr___spec__6___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -uint8_t x_13; -x_13 = lean_usize_dec_lt(x_4, x_3); -if (x_13 == 0) +lean_object* x_12; +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_1); +x_12 = l_Lean_Elab_realizeGlobalConstWithInfos(x_1, x_2, x_9, x_10, x_11); +if (lean_obj_tag(x_12) == 0) { -lean_object* x_14; -lean_dec(x_11); -lean_dec(x_10); +lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_dec(x_4); 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; +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_12, 1); +lean_inc(x_14); +lean_dec(x_12); +x_15 = lean_apply_8(x_3, x_13, x_5, x_6, x_7, x_8, x_9, x_10, x_14); +return x_15; } else { -lean_object* x_15; lean_object* x_16; -lean_dec(x_5); -x_15 = lean_array_uget(x_2, x_4); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_1); -x_16 = l_Lean_Attribute_erase(x_1, x_15, x_10, x_11, x_12); -if (lean_obj_tag(x_16) == 0) +uint8_t x_16; +x_16 = !lean_is_exclusive(x_12); +if (x_16 == 0) { -lean_object* x_17; size_t x_18; size_t x_19; lean_object* x_20; -x_17 = lean_ctor_get(x_16, 1); -lean_inc(x_17); -lean_dec(x_16); -x_18 = 1; -x_19 = lean_usize_add(x_4, x_18); -x_20 = lean_box(0); -x_4 = x_19; -x_5 = x_20; -x_12 = x_17; -goto _start; -} -else +lean_object* x_17; lean_object* x_18; uint8_t x_19; +x_17 = lean_ctor_get(x_12, 0); +x_18 = lean_ctor_get(x_12, 1); +x_19 = l_Lean_Exception_isInterrupt(x_17); +if (x_19 == 0) { -uint8_t x_22; -lean_dec(x_11); -lean_dec(x_10); +uint8_t x_20; +x_20 = l_Lean_Exception_isRuntime(x_17); +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_free_object(x_12); +lean_dec(x_17); +x_21 = l_Lean_Syntax_getId(x_1); lean_dec(x_1); -x_22 = !lean_is_exclusive(x_16); -if (x_22 == 0) +x_22 = lean_erase_macro_scopes(x_21); +x_23 = l_Lean_Meta_Simp_isBuiltinSimproc(x_22, x_9, x_10, x_18); +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_unbox(x_24); +lean_dec(x_24); +if (x_25 == 0) { -return x_16; +lean_object* x_26; lean_object* x_27; uint8_t x_28; +lean_dec(x_4); +lean_dec(x_3); +x_26 = lean_ctor_get(x_23, 1); +lean_inc(x_26); +lean_dec(x_23); +x_27 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabAttr___spec__5(x_22, x_5, x_6, x_7, x_8, x_9, x_10, x_26); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +x_28 = !lean_is_exclusive(x_27); +if (x_28 == 0) +{ +return x_27; } 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; -} -} -} +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_27, 0); +x_30 = lean_ctor_get(x_27, 1); +lean_inc(x_30); +lean_inc(x_29); +lean_dec(x_27); +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_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabAttr___spec__5___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("unknown constant '", 18, 18); -return x_1; -} -} -static lean_object* _init_l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabAttr___spec__5___closed__2() { -_start: +uint8_t x_32; +x_32 = !lean_is_exclusive(x_23); +if (x_32 == 0) { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabAttr___spec__5___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_23, 1); +x_34 = lean_ctor_get(x_23, 0); +lean_dec(x_34); +lean_ctor_set_tag(x_23, 1); +lean_ctor_set(x_23, 1, x_4); +lean_ctor_set(x_23, 0, x_22); +x_35 = lean_apply_8(x_3, x_23, x_5, x_6, x_7, x_8, x_9, x_10, x_33); +return x_35; } -static lean_object* _init_l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabAttr___spec__5___closed__3() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("'", 1, 1); -return x_1; +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_23, 1); +lean_inc(x_36); +lean_dec(x_23); +x_37 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_22); +lean_ctor_set(x_37, 1, x_4); +x_38 = lean_apply_8(x_3, x_37, x_5, x_6, x_7, x_8, x_9, x_10, x_36); +return x_38; } } -static lean_object* _init_l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabAttr___spec__5___closed__4() { -_start: +} +else { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabAttr___spec__5___closed__3; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +return x_12; } } -LEAN_EXPORT lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabAttr___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: +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; -x_9 = lean_box(0); -x_10 = l_Lean_Expr_const___override(x_1, x_9); -x_11 = l_Lean_MessageData_ofExpr(x_10); -x_12 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabAttr___spec__5___closed__2; -x_13 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_13, 0, x_12); -lean_ctor_set(x_13, 1, x_11); -x_14 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabAttr___spec__5___closed__4; -x_15 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_15, 0, x_13); -lean_ctor_set(x_15, 1, x_14); -x_16 = l_Lean_throwError___at_Lean_Elab_Term_expandDeclId___spec__11(x_15, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -return x_16; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +return x_12; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__6___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, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: +else { -lean_object* x_13; -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -x_13 = l_Lean_ensureNonAmbiguous___at_Lean_Elab_Command_elabAttr___spec__2(x_1, 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_39; lean_object* x_40; uint8_t x_41; +x_39 = lean_ctor_get(x_12, 0); +x_40 = lean_ctor_get(x_12, 1); +lean_inc(x_40); +lean_inc(x_39); +lean_dec(x_12); +x_41 = l_Lean_Exception_isInterrupt(x_39); +if (x_41 == 0) { -lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_14 = lean_ctor_get(x_13, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_13, 1); -lean_inc(x_15); -lean_dec(x_13); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_14); -x_16 = l_Lean_Elab_Term_applyAttributes(x_14, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_15); -if (lean_obj_tag(x_16) == 0) +uint8_t x_42; +x_42 = l_Lean_Exception_isRuntime(x_39); +if (x_42 == 0) { -lean_object* x_17; size_t 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 = lean_array_size(x_3); -x_19 = lean_box(0); -x_20 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__4(x_14, x_3, x_18, x_4, x_19, x_6, x_7, x_8, x_9, x_10, x_11, x_17); +lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; +lean_dec(x_39); +x_43 = l_Lean_Syntax_getId(x_1); +lean_dec(x_1); +x_44 = lean_erase_macro_scopes(x_43); +x_45 = l_Lean_Meta_Simp_isBuiltinSimproc(x_44, x_9, x_10, x_40); +x_46 = lean_ctor_get(x_45, 0); +lean_inc(x_46); +x_47 = lean_unbox(x_46); +lean_dec(x_46); +if (x_47 == 0) +{ +lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; +lean_dec(x_4); +lean_dec(x_3); +x_48 = lean_ctor_get(x_45, 1); +lean_inc(x_48); +lean_dec(x_45); +x_49 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabAttr___spec__5(x_44, x_5, x_6, x_7, x_8, x_9, x_10, x_48); +lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -if (lean_obj_tag(x_20) == 0) -{ -uint8_t x_21; -x_21 = !lean_is_exclusive(x_20); -if (x_21 == 0) -{ -lean_object* x_22; -x_22 = lean_ctor_get(x_20, 0); -lean_dec(x_22); -lean_ctor_set(x_20, 0, x_19); -return x_20; +x_50 = lean_ctor_get(x_49, 0); +lean_inc(x_50); +x_51 = lean_ctor_get(x_49, 1); +lean_inc(x_51); +if (lean_is_exclusive(x_49)) { + lean_ctor_release(x_49, 0); + lean_ctor_release(x_49, 1); + x_52 = x_49; +} else { + lean_dec_ref(x_49); + x_52 = lean_box(0); } -else -{ -lean_object* x_23; lean_object* x_24; -x_23 = lean_ctor_get(x_20, 1); -lean_inc(x_23); -lean_dec(x_20); -x_24 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_24, 0, x_19); -lean_ctor_set(x_24, 1, x_23); -return x_24; +if (lean_is_scalar(x_52)) { + x_53 = lean_alloc_ctor(1, 2, 0); +} else { + x_53 = x_52; } +lean_ctor_set(x_53, 0, x_50); +lean_ctor_set(x_53, 1, x_51); +return x_53; } else { -uint8_t x_25; -x_25 = !lean_is_exclusive(x_20); -if (x_25 == 0) -{ -return x_20; +lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_54 = lean_ctor_get(x_45, 1); +lean_inc(x_54); +if (lean_is_exclusive(x_45)) { + lean_ctor_release(x_45, 0); + lean_ctor_release(x_45, 1); + x_55 = x_45; +} else { + lean_dec_ref(x_45); + x_55 = lean_box(0); } -else -{ -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_20, 0); -x_27 = lean_ctor_get(x_20, 1); -lean_inc(x_27); -lean_inc(x_26); -lean_dec(x_20); -x_28 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_28, 0, x_26); -lean_ctor_set(x_28, 1, x_27); -return x_28; +if (lean_is_scalar(x_55)) { + x_56 = lean_alloc_ctor(1, 2, 0); +} else { + x_56 = x_55; + lean_ctor_set_tag(x_56, 1); } +lean_ctor_set(x_56, 0, x_44); +lean_ctor_set(x_56, 1, x_4); +x_57 = lean_apply_8(x_3, x_56, x_5, x_6, x_7, x_8, x_9, x_10, x_54); +return x_57; } } else { -uint8_t x_29; -lean_dec(x_14); -lean_dec(x_11); +lean_object* x_58; lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -x_29 = !lean_is_exclusive(x_16); -if (x_29 == 0) -{ -return x_16; -} -else -{ -lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_30 = lean_ctor_get(x_16, 0); -x_31 = lean_ctor_get(x_16, 1); -lean_inc(x_31); -lean_inc(x_30); -lean_dec(x_16); -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_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_58 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_58, 0, x_39); +lean_ctor_set(x_58, 1, x_40); +return x_58; } } else { -uint8_t x_33; -lean_dec(x_11); +lean_object* x_59; lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_2); -x_33 = !lean_is_exclusive(x_13); -if (x_33 == 0) +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_59 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_59, 0, x_39); +lean_ctor_set(x_59, 1, x_40); +return x_59; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__6(lean_object* x_1, size_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, size_t x_6, size_t x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +uint8_t x_12; +x_12 = lean_usize_dec_lt(x_7, x_6); +if (x_12 == 0) { +lean_object* x_13; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_8); +lean_ctor_set(x_13, 1, x_11); return x_13; } else { -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_13, 0); -x_35 = lean_ctor_get(x_13, 1); +lean_object* x_14; lean_object* x_15; lean_object* x_16; 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; uint8_t x_32; lean_object* x_33; lean_object* x_34; +lean_dec(x_8); +x_14 = lean_array_uget(x_5, x_7); +x_15 = lean_box_usize(x_2); +lean_inc(x_3); +lean_inc(x_4); +lean_inc(x_14); +x_16 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__6___lambda__1___boxed), 12, 4); +lean_closure_set(x_16, 0, x_14); +lean_closure_set(x_16, 1, x_4); +lean_closure_set(x_16, 2, x_3); +lean_closure_set(x_16, 3, x_15); +x_17 = lean_box(0); +lean_inc(x_1); +lean_inc(x_14); +x_18 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__6___lambda__2), 11, 4); +lean_closure_set(x_18, 0, x_14); +lean_closure_set(x_18, 1, x_17); +lean_closure_set(x_18, 2, x_16); +lean_closure_set(x_18, 3, x_1); +x_19 = l_Lean_Elab_Command_getRef(x_9, x_10, x_11); +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_replaceRef(x_14, x_20); +lean_dec(x_20); +lean_dec(x_14); +x_23 = lean_ctor_get(x_9, 0); +x_24 = lean_ctor_get(x_9, 1); +x_25 = lean_ctor_get(x_9, 2); +x_26 = lean_ctor_get(x_9, 3); +x_27 = lean_ctor_get(x_9, 4); +x_28 = lean_ctor_get(x_9, 5); +x_29 = lean_ctor_get(x_9, 7); +x_30 = lean_ctor_get(x_9, 8); +x_31 = lean_ctor_get(x_9, 9); +x_32 = lean_ctor_get_uint8(x_9, sizeof(void*)*10); +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); +x_33 = lean_alloc_ctor(0, 10, 1); +lean_ctor_set(x_33, 0, x_23); +lean_ctor_set(x_33, 1, x_24); +lean_ctor_set(x_33, 2, x_25); +lean_ctor_set(x_33, 3, x_26); +lean_ctor_set(x_33, 4, x_27); +lean_ctor_set(x_33, 5, x_28); +lean_ctor_set(x_33, 6, x_22); +lean_ctor_set(x_33, 7, x_29); +lean_ctor_set(x_33, 8, x_30); +lean_ctor_set(x_33, 9, x_31); +lean_ctor_set_uint8(x_33, sizeof(void*)*10, x_32); +x_34 = l_Lean_Elab_Command_liftTermElabM___rarg(x_18, x_33, x_10, x_21); +lean_dec(x_33); +if (lean_obj_tag(x_34) == 0) +{ +lean_object* x_35; size_t x_36; size_t x_37; lean_object* x_38; +x_35 = lean_ctor_get(x_34, 1); lean_inc(x_35); -lean_inc(x_34); -lean_dec(x_13); -x_36 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_36, 0, x_34); -lean_ctor_set(x_36, 1, x_35); -return x_36; +lean_dec(x_34); +x_36 = 1; +x_37 = lean_usize_add(x_7, x_36); +x_38 = lean_box(0); +x_7 = x_37; +x_8 = x_38; +x_11 = x_35; +goto _start; +} +else +{ +uint8_t x_40; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_40 = !lean_is_exclusive(x_34); +if (x_40 == 0) +{ +return x_34; } +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); +lean_inc(x_42); +lean_inc(x_41); +lean_dec(x_34); +x_43 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_43, 0, x_41); +lean_ctor_set(x_43, 1, x_42); +return x_43; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__6___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +} +} +static lean_object* _init_l_Lean_Elab_Command_elabAttr___closed__1() { _start: { -lean_object* x_12; -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_1); -x_12 = l_Lean_Elab_realizeGlobalConstWithInfos(x_1, x_2, x_9, x_10, x_11); -if (lean_obj_tag(x_12) == 0) +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__4; +x_2 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_2, 0, x_1); +lean_ctor_set(x_2, 1, x_1); +return x_2; +} +} +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_13; lean_object* x_14; lean_object* x_15; -lean_dec(x_4); -lean_dec(x_1); +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_box(0); +x_6 = lean_unsigned_to_nat(2u); +x_7 = l_Lean_Syntax_getArg(x_1, x_6); +x_8 = l_Lean_Syntax_getSepArgs(x_7); +lean_dec(x_7); +x_9 = lean_array_size(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_8, x_9, x_10, x_11, x_2, x_3, x_4); +lean_dec(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 = lean_apply_8(x_3, x_13, x_5, x_6, x_7, x_8, x_9, x_10, x_14); -return x_15; -} -else -{ -uint8_t x_16; -x_16 = !lean_is_exclusive(x_12); -if (x_16 == 0) +x_15 = lean_ctor_get(x_13, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_13, 1); +lean_inc(x_16); +lean_dec(x_13); +lean_inc(x_2); +x_17 = l_Lean_Elab_elabAttrs___at_Lean_Elab_Command_elabMutualDef___spec__3(x_15, x_2, x_3, x_14); +lean_dec(x_15); +if (lean_obj_tag(x_17) == 0) { -lean_object* x_17; lean_object* x_18; uint8_t x_19; -x_17 = lean_ctor_get(x_12, 0); -x_18 = lean_ctor_get(x_12, 1); -x_19 = l_Lean_Exception_isInterrupt(x_17); -if (x_19 == 0) +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; size_t x_23; lean_object* x_24; lean_object* x_25; +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_unsigned_to_nat(4u); +x_21 = l_Lean_Syntax_getArg(x_1, x_20); +x_22 = l_Lean_Syntax_getArgs(x_21); +lean_dec(x_21); +x_23 = lean_array_size(x_22); +x_24 = lean_box(0); +x_25 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__6(x_5, x_10, x_16, x_18, x_22, x_23, x_10, x_24, x_2, x_3, x_19); +lean_dec(x_2); +lean_dec(x_22); +if (lean_obj_tag(x_25) == 0) { -uint8_t x_20; -x_20 = l_Lean_Exception_isRuntime(x_17); -if (x_20 == 0) +uint8_t x_26; +x_26 = !lean_is_exclusive(x_25); +if (x_26 == 0) { -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; -lean_free_object(x_12); -lean_dec(x_17); -x_21 = l_Lean_Syntax_getId(x_1); -lean_dec(x_1); -x_22 = lean_erase_macro_scopes(x_21); -x_23 = l_Lean_Meta_Simp_isBuiltinSimproc(x_22, x_9, x_10, x_18); -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -x_25 = lean_unbox(x_24); -lean_dec(x_24); -if (x_25 == 0) +lean_object* x_27; +x_27 = lean_ctor_get(x_25, 0); +lean_dec(x_27); +lean_ctor_set(x_25, 0, x_24); +return x_25; +} +else { -lean_object* x_26; lean_object* x_27; uint8_t x_28; -lean_dec(x_4); -lean_dec(x_3); -x_26 = lean_ctor_get(x_23, 1); -lean_inc(x_26); -lean_dec(x_23); -x_27 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabAttr___spec__5(x_22, x_5, x_6, x_7, x_8, x_9, x_10, x_26); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -x_28 = !lean_is_exclusive(x_27); -if (x_28 == 0) +lean_object* x_28; lean_object* x_29; +x_28 = lean_ctor_get(x_25, 1); +lean_inc(x_28); +lean_dec(x_25); +x_29 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_29, 0, x_24); +lean_ctor_set(x_29, 1, x_28); +return x_29; +} +} +else { -return x_27; +uint8_t x_30; +x_30 = !lean_is_exclusive(x_25); +if (x_30 == 0) +{ +return x_25; } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_27, 0); -x_30 = lean_ctor_get(x_27, 1); -lean_inc(x_30); -lean_inc(x_29); -lean_dec(x_27); -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_31; lean_object* x_32; lean_object* x_33; +x_31 = lean_ctor_get(x_25, 0); +x_32 = lean_ctor_get(x_25, 1); +lean_inc(x_32); +lean_inc(x_31); +lean_dec(x_25); +x_33 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_33, 0, x_31); +lean_ctor_set(x_33, 1, x_32); +return x_33; +} } } else { -uint8_t x_32; -x_32 = !lean_is_exclusive(x_23); -if (x_32 == 0) +uint8_t x_34; +lean_dec(x_16); +lean_dec(x_2); +x_34 = !lean_is_exclusive(x_17); +if (x_34 == 0) { -lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_33 = lean_ctor_get(x_23, 1); -x_34 = lean_ctor_get(x_23, 0); -lean_dec(x_34); -lean_ctor_set_tag(x_23, 1); -lean_ctor_set(x_23, 1, x_4); -lean_ctor_set(x_23, 0, x_22); -x_35 = lean_apply_8(x_3, x_23, x_5, x_6, x_7, x_8, x_9, x_10, x_33); -return x_35; +return x_17; } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_23, 1); +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_dec(x_23); +lean_inc(x_35); +lean_dec(x_17); x_37 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_37, 0, x_22); -lean_ctor_set(x_37, 1, x_4); -x_38 = lean_apply_8(x_3, x_37, x_5, x_6, x_7, x_8, x_9, x_10, x_36); -return x_38; +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +return x_37; } } } -else +} +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: { -lean_dec(x_10); +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_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_1); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___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) { +_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_Command_elabAttr___spec__4(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); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); +lean_dec(x_2); +return x_15; +} +} +LEAN_EXPORT lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabAttr___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +x_9 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabAttr___spec__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_7); +lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_1); -return x_12; +return x_9; } } -else +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___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_object* x_12) { +_start: +{ +size_t x_13; lean_object* x_14; +x_13 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_14 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__6___lambda__1(x_1, x_2, x_3, x_13, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_3); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___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) { +_start: { +size_t x_12; size_t x_13; size_t x_14; lean_object* x_15; +x_12 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_13 = lean_unbox_usize(x_6); +lean_dec(x_6); +x_14 = lean_unbox_usize(x_7); +lean_dec(x_7); +x_15 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__6(x_1, x_12, x_3, x_4, x_5, x_13, x_14, 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_15; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAttr___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Lean_Elab_Command_elabAttr(x_1, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_1); -return x_12; +return x_5; } } -else +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabAttr__1___closed__1() { +_start: { -lean_object* x_39; lean_object* x_40; uint8_t x_41; -x_39 = lean_ctor_get(x_12, 0); -x_40 = lean_ctor_get(x_12, 1); -lean_inc(x_40); -lean_inc(x_39); -lean_dec(x_12); -x_41 = l_Lean_Exception_isInterrupt(x_39); -if (x_41 == 0) +lean_object* x_1; +x_1 = lean_mk_string_unchecked("attribute", 9, 9); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabAttr__1___closed__2() { +_start: { -uint8_t x_42; -x_42 = l_Lean_Exception_isRuntime(x_39); -if (x_42 == 0) +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__1; +x_2 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__2; +x_3 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__3; +x_4 = l___regBuiltin_Lean_Elab_Command_elabAttr__1___closed__1; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabAttr__1___closed__3() { +_start: { -lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; -lean_dec(x_39); -x_43 = l_Lean_Syntax_getId(x_1); -lean_dec(x_1); -x_44 = lean_erase_macro_scopes(x_43); -x_45 = l_Lean_Meta_Simp_isBuiltinSimproc(x_44, x_9, x_10, x_40); -x_46 = lean_ctor_get(x_45, 0); -lean_inc(x_46); -x_47 = lean_unbox(x_46); -lean_dec(x_46); -if (x_47 == 0) +lean_object* x_1; +x_1 = lean_mk_string_unchecked("elabAttr", 8, 8); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabAttr__1___closed__4() { +_start: { -lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; -lean_dec(x_4); -lean_dec(x_3); -x_48 = lean_ctor_get(x_45, 1); -lean_inc(x_48); -lean_dec(x_45); -x_49 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabAttr___spec__5(x_44, x_5, x_6, x_7, x_8, x_9, x_10, x_48); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -x_50 = lean_ctor_get(x_49, 0); -lean_inc(x_50); -x_51 = lean_ctor_get(x_49, 1); -lean_inc(x_51); -if (lean_is_exclusive(x_49)) { - lean_ctor_release(x_49, 0); - lean_ctor_release(x_49, 1); - x_52 = x_49; -} else { - lean_dec_ref(x_49); - x_52 = lean_box(0); +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__1; +x_2 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__6; +x_3 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__3; +x_4 = l___regBuiltin_Lean_Elab_Command_elabAttr__1___closed__3; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; } -if (lean_is_scalar(x_52)) { - x_53 = lean_alloc_ctor(1, 2, 0); -} else { - x_53 = x_52; } -lean_ctor_set(x_53, 0, x_50); -lean_ctor_set(x_53, 1, x_51); -return x_53; +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabAttr__1___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabAttr___boxed), 4, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabAttr__1(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Elab_Command_elabDeclaration__1___closed__3; +x_3 = l___regBuiltin_Lean_Elab_Command_elabAttr__1___closed__2; +x_4 = l___regBuiltin_Lean_Elab_Command_elabAttr__1___closed__4; +x_5 = l___regBuiltin_Lean_Elab_Command_elabAttr__1___closed__5; +x_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_elabAttr_declRange__1___closed__1() { +_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(36u); +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; +} } -else +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1___closed__2() { +_start: { -lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; -x_54 = lean_ctor_get(x_45, 1); -lean_inc(x_54); -if (lean_is_exclusive(x_45)) { - lean_ctor_release(x_45, 0); - lean_ctor_release(x_45, 1); - x_55 = x_45; -} else { - lean_dec_ref(x_45); - x_55 = lean_box(0); +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_unsigned_to_nat(383u); +x_2 = lean_unsigned_to_nat(39u); +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; } -if (lean_is_scalar(x_55)) { - x_56 = lean_alloc_ctor(1, 2, 0); -} else { - x_56 = x_55; - lean_ctor_set_tag(x_56, 1); } -lean_ctor_set(x_56, 0, x_44); -lean_ctor_set(x_56, 1, x_4); -x_57 = lean_apply_8(x_3, x_56, x_5, x_6, x_7, x_8, x_9, x_10, x_54); -return x_57; +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1___closed__1; +x_2 = lean_unsigned_to_nat(36u); +x_3 = l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1___closed__2; +x_4 = lean_unsigned_to_nat(39u); +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; } } -else +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1___closed__4() { +_start: { -lean_object* x_58; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_58 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_58, 0, x_39); -lean_ctor_set(x_58, 1, x_40); -return x_58; +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(40u); +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; } } -else +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1___closed__5() { +_start: { -lean_object* x_59; -lean_dec(x_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_59 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_59, 0, x_39); -lean_ctor_set(x_59, 1, x_40); -return x_59; +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(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; +} } +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1___closed__4; +x_2 = lean_unsigned_to_nat(40u); +x_3 = l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1___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; } } +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1___closed__3; +x_2 = l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__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; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__6(lean_object* x_1, size_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, size_t x_6, size_t x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1(lean_object* x_1) { _start: { -uint8_t x_12; -x_12 = lean_usize_dec_lt(x_7, x_6); -if (x_12 == 0) +lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_2 = l___regBuiltin_Lean_Elab_Command_elabAttr__1___closed__4; +x_3 = l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1___closed__7; +x_4 = l_Lean_addBuiltinDeclarationRanges(x_2, x_3, x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Command_elabInitialize___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: { -lean_object* x_13; -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_8); -lean_ctor_set(x_13, 1, x_11); -return x_13; +uint8_t x_5; lean_object* x_6; +x_5 = 0; +x_6 = l_Lean_Syntax_getRange_x3f(x_1, x_5); +if (lean_obj_tag(x_6) == 0) +{ +lean_object* x_7; lean_object* x_8; +lean_dec(x_2); +x_7 = lean_box(0); +x_8 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_8, 0, x_7); +lean_ctor_set(x_8, 1, x_4); +return x_8; } else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; 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; uint8_t x_32; lean_object* x_33; lean_object* x_34; -lean_dec(x_8); -x_14 = lean_array_uget(x_5, x_7); -x_15 = lean_box_usize(x_2); -lean_inc(x_3); -lean_inc(x_4); -lean_inc(x_14); -x_16 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__6___lambda__1___boxed), 12, 4); -lean_closure_set(x_16, 0, x_14); -lean_closure_set(x_16, 1, x_4); -lean_closure_set(x_16, 2, x_3); -lean_closure_set(x_16, 3, x_15); -x_17 = lean_box(0); -lean_inc(x_1); +uint8_t x_9; +x_9 = !lean_is_exclusive(x_6); +if (x_9 == 0) +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_10 = lean_ctor_get(x_6, 0); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); +lean_dec(x_2); +x_12 = lean_ctor_get(x_10, 0); +lean_inc(x_12); +lean_inc(x_11); +x_13 = l_Lean_FileMap_toPosition(x_11, x_12); +lean_dec(x_12); +x_14 = lean_ctor_get(x_10, 1); lean_inc(x_14); -x_18 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__6___lambda__2), 11, 4); -lean_closure_set(x_18, 0, x_14); -lean_closure_set(x_18, 1, x_17); -lean_closure_set(x_18, 2, x_16); -lean_closure_set(x_18, 3, x_1); -x_19 = l_Lean_Elab_Command_getRef(x_9, x_10, x_11); -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_replaceRef(x_14, x_20); -lean_dec(x_20); +lean_dec(x_10); +lean_inc(x_11); +x_15 = l_Lean_FileMap_toPosition(x_11, x_14); lean_dec(x_14); -x_23 = lean_ctor_get(x_9, 0); -x_24 = lean_ctor_get(x_9, 1); -x_25 = lean_ctor_get(x_9, 2); -x_26 = lean_ctor_get(x_9, 3); -x_27 = lean_ctor_get(x_9, 4); -x_28 = lean_ctor_get(x_9, 5); -x_29 = lean_ctor_get(x_9, 7); -x_30 = lean_ctor_get(x_9, 8); -x_31 = lean_ctor_get(x_9, 9); -x_32 = lean_ctor_get_uint8(x_9, sizeof(void*)*10); -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); -x_33 = lean_alloc_ctor(0, 10, 1); -lean_ctor_set(x_33, 0, x_23); -lean_ctor_set(x_33, 1, x_24); -lean_ctor_set(x_33, 2, x_25); -lean_ctor_set(x_33, 3, x_26); -lean_ctor_set(x_33, 4, x_27); -lean_ctor_set(x_33, 5, x_28); -lean_ctor_set(x_33, 6, x_22); -lean_ctor_set(x_33, 7, x_29); -lean_ctor_set(x_33, 8, x_30); -lean_ctor_set(x_33, 9, x_31); -lean_ctor_set_uint8(x_33, sizeof(void*)*10, x_32); -x_34 = l_Lean_Elab_Command_liftTermElabM___rarg(x_18, x_33, x_10, x_21); -lean_dec(x_33); -if (lean_obj_tag(x_34) == 0) +lean_inc(x_13); +x_16 = l_Lean_FileMap_leanPosToLspPos(x_11, x_13); +x_17 = !lean_is_exclusive(x_16); +if (x_17 == 0) { -lean_object* x_35; size_t x_36; size_t x_37; lean_object* x_38; -x_35 = lean_ctor_get(x_34, 1); -lean_inc(x_35); -lean_dec(x_34); -x_36 = 1; -x_37 = lean_usize_add(x_7, x_36); -x_38 = lean_box(0); -x_7 = x_37; -x_8 = x_38; -x_11 = x_35; -goto _start; +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_18 = lean_ctor_get(x_16, 1); +x_19 = lean_ctor_get(x_16, 0); +lean_dec(x_19); +lean_inc(x_15); +x_20 = l_Lean_FileMap_leanPosToLspPos(x_11, x_15); +lean_dec(x_11); +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +x_22 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_22, 0, x_13); +lean_ctor_set(x_22, 1, x_18); +lean_ctor_set(x_22, 2, x_15); +lean_ctor_set(x_22, 3, x_21); +lean_ctor_set(x_6, 0, x_22); +lean_ctor_set(x_16, 1, x_4); +lean_ctor_set(x_16, 0, x_6); +return x_16; } else { -uint8_t x_40; -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_40 = !lean_is_exclusive(x_34); -if (x_40 == 0) -{ -return x_34; +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); +lean_inc(x_15); +x_24 = l_Lean_FileMap_leanPosToLspPos(x_11, x_15); +lean_dec(x_11); +x_25 = lean_ctor_get(x_24, 1); +lean_inc(x_25); +lean_dec(x_24); +x_26 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_26, 0, x_13); +lean_ctor_set(x_26, 1, x_23); +lean_ctor_set(x_26, 2, x_15); +lean_ctor_set(x_26, 3, x_25); +lean_ctor_set(x_6, 0, x_26); +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_6); +lean_ctor_set(x_27, 1, x_4); +return x_27; +} } else { -lean_object* x_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); -lean_inc(x_42); -lean_inc(x_41); -lean_dec(x_34); -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_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_28 = lean_ctor_get(x_6, 0); +lean_inc(x_28); +lean_dec(x_6); +x_29 = lean_ctor_get(x_2, 1); +lean_inc(x_29); +lean_dec(x_2); +x_30 = lean_ctor_get(x_28, 0); +lean_inc(x_30); +lean_inc(x_29); +x_31 = l_Lean_FileMap_toPosition(x_29, x_30); +lean_dec(x_30); +x_32 = lean_ctor_get(x_28, 1); +lean_inc(x_32); +lean_dec(x_28); +lean_inc(x_29); +x_33 = l_Lean_FileMap_toPosition(x_29, x_32); +lean_dec(x_32); +lean_inc(x_31); +x_34 = l_Lean_FileMap_leanPosToLspPos(x_29, x_31); +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); +} +lean_inc(x_33); +x_37 = l_Lean_FileMap_leanPosToLspPos(x_29, x_33); +lean_dec(x_29); +x_38 = lean_ctor_get(x_37, 1); +lean_inc(x_38); +lean_dec(x_37); +x_39 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_39, 0, x_31); +lean_ctor_set(x_39, 1, x_35); +lean_ctor_set(x_39, 2, x_33); +lean_ctor_set(x_39, 3, x_38); +x_40 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_40, 0, x_39); +if (lean_is_scalar(x_36)) { + x_41 = lean_alloc_ctor(0, 2, 0); +} else { + x_41 = x_36; } +lean_ctor_set(x_41, 0, x_40); +lean_ctor_set(x_41, 1, x_4); +return x_41; } } } } -static lean_object* _init_l_Lean_Elab_Command_elabAttr___closed__1() { +static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabInitialize___spec__4___closed__1() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__4; -x_2 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_2, 0, x_1); -lean_ctor_set(x_2, 1, x_1); -return x_2; +lean_object* x_1; +x_1 = l_Lean_declRangeExt; +return x_1; } } -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) { +LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabInitialize___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_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_box(0); -x_6 = lean_unsigned_to_nat(2u); -x_7 = l_Lean_Syntax_getArg(x_1, x_6); -x_8 = l_Lean_Syntax_getSepArgs(x_7); -lean_dec(x_7); -x_9 = lean_array_size(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_8, x_9, x_10, x_11, x_2, x_3, x_4); +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; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_8 = lean_ctor_get(x_6, 0); +x_9 = lean_ctor_get(x_6, 1); +x_10 = lean_ctor_get(x_8, 0); +lean_inc(x_10); lean_dec(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 = lean_ctor_get(x_13, 0); +x_11 = l_Lean_instInhabitedDeclarationRanges; +x_12 = l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabInitialize___spec__4___closed__1; +lean_inc(x_1); +x_13 = l_Lean_MapDeclarationExtension_contains___rarg(x_11, x_12, x_10, x_1); +lean_dec(x_10); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +lean_free_object(x_6); +x_14 = lean_st_ref_take(x_4, x_9); +x_15 = lean_ctor_get(x_14, 0); lean_inc(x_15); -x_16 = lean_ctor_get(x_13, 1); +x_16 = lean_ctor_get(x_14, 1); lean_inc(x_16); -lean_dec(x_13); -lean_inc(x_2); -x_17 = l_Lean_Elab_elabAttrs___at_Lean_Elab_Command_elabMutualDef___spec__3(x_15, x_2, x_3, x_14); -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; size_t x_23; lean_object* x_24; lean_object* x_25; -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_unsigned_to_nat(4u); -x_21 = l_Lean_Syntax_getArg(x_1, x_20); -x_22 = l_Lean_Syntax_getArgs(x_21); -lean_dec(x_21); -x_23 = lean_array_size(x_22); -x_24 = lean_box(0); -x_25 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__6(x_5, x_10, x_16, x_18, x_22, x_23, x_10, x_24, x_2, x_3, x_19); -lean_dec(x_2); -lean_dec(x_22); -if (lean_obj_tag(x_25) == 0) +lean_dec(x_14); +x_17 = !lean_is_exclusive(x_15); +if (x_17 == 0) { -uint8_t x_26; -x_26 = !lean_is_exclusive(x_25); -if (x_26 == 0) +lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_18 = lean_ctor_get(x_15, 0); +x_19 = l_Lean_MapDeclarationExtension_insert___rarg(x_12, x_18, x_1, x_2); +lean_ctor_set(x_15, 0, x_19); +x_20 = lean_st_ref_set(x_4, x_15, x_16); +x_21 = !lean_is_exclusive(x_20); +if (x_21 == 0) { -lean_object* x_27; -x_27 = lean_ctor_get(x_25, 0); -lean_dec(x_27); -lean_ctor_set(x_25, 0, x_24); -return x_25; +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_28; lean_object* x_29; -x_28 = lean_ctor_get(x_25, 1); -lean_inc(x_28); -lean_dec(x_25); -x_29 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_29, 0, x_24); -lean_ctor_set(x_29, 1, x_28); -return x_29; -} +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 -{ -uint8_t x_30; -x_30 = !lean_is_exclusive(x_25); -if (x_30 == 0) -{ -return x_25; } else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_31 = lean_ctor_get(x_25, 0); -x_32 = lean_ctor_get(x_25, 1); +lean_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; +x_27 = lean_ctor_get(x_15, 0); +x_28 = lean_ctor_get(x_15, 1); +x_29 = lean_ctor_get(x_15, 2); +x_30 = lean_ctor_get(x_15, 3); +x_31 = lean_ctor_get(x_15, 4); +x_32 = lean_ctor_get(x_15, 5); +x_33 = lean_ctor_get(x_15, 6); +x_34 = lean_ctor_get(x_15, 7); +lean_inc(x_34); +lean_inc(x_33); lean_inc(x_32); lean_inc(x_31); -lean_dec(x_25); -x_33 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_33, 0, x_31); -lean_ctor_set(x_33, 1, x_32); -return x_33; +lean_inc(x_30); +lean_inc(x_29); +lean_inc(x_28); +lean_inc(x_27); +lean_dec(x_15); +x_35 = l_Lean_MapDeclarationExtension_insert___rarg(x_12, x_27, x_1, x_2); +x_36 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_36, 0, x_35); +lean_ctor_set(x_36, 1, x_28); +lean_ctor_set(x_36, 2, x_29); +lean_ctor_set(x_36, 3, x_30); +lean_ctor_set(x_36, 4, x_31); +lean_ctor_set(x_36, 5, x_32); +lean_ctor_set(x_36, 6, x_33); +lean_ctor_set(x_36, 7, x_34); +x_37 = lean_st_ref_set(x_4, x_36, x_16); +x_38 = lean_ctor_get(x_37, 1); +lean_inc(x_38); +if (lean_is_exclusive(x_37)) { + lean_ctor_release(x_37, 0); + lean_ctor_release(x_37, 1); + x_39 = x_37; +} else { + lean_dec_ref(x_37); + x_39 = lean_box(0); +} +x_40 = lean_box(0); +if (lean_is_scalar(x_39)) { + x_41 = lean_alloc_ctor(0, 2, 0); +} else { + x_41 = x_39; } +lean_ctor_set(x_41, 0, x_40); +lean_ctor_set(x_41, 1, x_38); +return x_41; } } else { -uint8_t x_34; -lean_dec(x_16); +lean_object* x_42; lean_dec(x_2); -x_34 = !lean_is_exclusive(x_17); -if (x_34 == 0) +lean_dec(x_1); +x_42 = lean_box(0); +lean_ctor_set(x_6, 0, x_42); +return x_6; +} +} +else { -return x_17; +lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; +x_43 = lean_ctor_get(x_6, 0); +x_44 = lean_ctor_get(x_6, 1); +lean_inc(x_44); +lean_inc(x_43); +lean_dec(x_6); +x_45 = lean_ctor_get(x_43, 0); +lean_inc(x_45); +lean_dec(x_43); +x_46 = l_Lean_instInhabitedDeclarationRanges; +x_47 = l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabInitialize___spec__4___closed__1; +lean_inc(x_1); +x_48 = l_Lean_MapDeclarationExtension_contains___rarg(x_46, x_47, x_45, x_1); +lean_dec(x_45); +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; +x_49 = lean_st_ref_take(x_4, 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 = lean_ctor_get(x_50, 0); +lean_inc(x_52); +x_53 = lean_ctor_get(x_50, 1); +lean_inc(x_53); +x_54 = lean_ctor_get(x_50, 2); +lean_inc(x_54); +x_55 = lean_ctor_get(x_50, 3); +lean_inc(x_55); +x_56 = lean_ctor_get(x_50, 4); +lean_inc(x_56); +x_57 = lean_ctor_get(x_50, 5); +lean_inc(x_57); +x_58 = lean_ctor_get(x_50, 6); +lean_inc(x_58); +x_59 = lean_ctor_get(x_50, 7); +lean_inc(x_59); +if (lean_is_exclusive(x_50)) { + lean_ctor_release(x_50, 0); + lean_ctor_release(x_50, 1); + lean_ctor_release(x_50, 2); + lean_ctor_release(x_50, 3); + lean_ctor_release(x_50, 4); + lean_ctor_release(x_50, 5); + lean_ctor_release(x_50, 6); + lean_ctor_release(x_50, 7); + x_60 = x_50; +} else { + lean_dec_ref(x_50); + x_60 = lean_box(0); } -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; +x_61 = l_Lean_MapDeclarationExtension_insert___rarg(x_47, x_52, x_1, x_2); +if (lean_is_scalar(x_60)) { + x_62 = lean_alloc_ctor(0, 8, 0); +} else { + x_62 = x_60; } +lean_ctor_set(x_62, 0, x_61); +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_56); +lean_ctor_set(x_62, 5, x_57); +lean_ctor_set(x_62, 6, x_58); +lean_ctor_set(x_62, 7, x_59); +x_63 = lean_st_ref_set(x_4, x_62, x_51); +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_box(0); +if (lean_is_scalar(x_65)) { + x_67 = lean_alloc_ctor(0, 2, 0); +} else { + x_67 = x_65; } +lean_ctor_set(x_67, 0, x_66); +lean_ctor_set(x_67, 1, x_64); +return x_67; } -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: +else { -size_t x_8; size_t x_9; lean_object* x_10; -x_8 = lean_unbox_usize(x_2); +lean_object* x_68; lean_object* x_69; lean_dec(x_2); -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_1); -return x_10; +x_68 = lean_box(0); +x_69 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_69, 0, x_68); +lean_ctor_set(x_69, 1, x_44); +return x_69; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___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) { -_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_Command_elabAttr___spec__4(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); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_2); -return x_15; } } -LEAN_EXPORT lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabAttr___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___at_Lean_Elab_Command_elabInitialize___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { -lean_object* x_9; -x_9 = l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabAttr___spec__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_7); -lean_dec(x_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_Command_elabAttr___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_object* x_12) { -_start: +lean_object* x_7; lean_object* x_8; +lean_inc(x_4); +x_7 = l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Command_elabInitialize___spec__3(x_2, x_4, x_5, x_6); +x_8 = lean_ctor_get(x_7, 0); +lean_inc(x_8); +if (lean_obj_tag(x_8) == 0) { -size_t x_13; lean_object* x_14; -x_13 = lean_unbox_usize(x_4); +uint8_t x_9; lean_dec(x_4); -x_14 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__6___lambda__1(x_1, x_2, x_3, x_13, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_3); -return x_14; -} -} -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___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) { -_start: +lean_dec(x_1); +x_9 = !lean_is_exclusive(x_7); +if (x_9 == 0) { -size_t x_12; size_t x_13; size_t x_14; lean_object* x_15; -x_12 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_13 = lean_unbox_usize(x_6); -lean_dec(x_6); -x_14 = lean_unbox_usize(x_7); -lean_dec(x_7); -x_15 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__6(x_1, x_12, x_3, x_4, x_5, x_13, x_14, x_8, x_9, x_10, x_11); +lean_object* x_10; lean_object* x_11; +x_10 = lean_ctor_get(x_7, 0); lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_5); -return x_15; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAttr___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -lean_object* x_5; -x_5 = l_Lean_Elab_Command_elabAttr(x_1, x_2, x_3, x_4); -lean_dec(x_3); -lean_dec(x_1); -return x_5; -} +x_11 = lean_box(0); +lean_ctor_set(x_7, 0, x_11); +return x_7; } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabAttr__1___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("attribute", 9, 9); -return x_1; +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_7, 1); +lean_inc(x_12); +lean_dec(x_7); +x_13 = lean_box(0); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_13); +lean_ctor_set(x_14, 1, x_12); +return x_14; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabAttr__1___closed__2() { -_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___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__1; -x_2 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__2; -x_3 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__3; -x_4 = l___regBuiltin_Lean_Elab_Command_elabAttr__1___closed__1; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabAttr__1___closed__3() { -_start: +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_15 = lean_ctor_get(x_7, 1); +lean_inc(x_15); +lean_dec(x_7); +x_16 = lean_ctor_get(x_8, 0); +lean_inc(x_16); +lean_dec(x_8); +lean_inc(x_4); +x_17 = l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Command_elabInitialize___spec__3(x_3, x_4, x_5, x_15); +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +if (lean_obj_tag(x_18) == 0) { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("elabAttr", 8, 8); -return x_1; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabAttr__1___closed__4() { -_start: +uint8_t x_19; +x_19 = !lean_is_exclusive(x_17); +if (x_19 == 0) { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__1; -x_2 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__6; -x_3 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__3; -x_4 = l___regBuiltin_Lean_Elab_Command_elabAttr__1___closed__3; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; -} +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_17, 1); +x_21 = lean_ctor_get(x_17, 0); +lean_dec(x_21); +lean_inc(x_16); +lean_ctor_set(x_17, 1, x_16); +lean_ctor_set(x_17, 0, x_16); +x_22 = l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabInitialize___spec__4(x_1, x_17, x_4, x_5, x_20); +lean_dec(x_4); +return x_22; } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabAttr__1___closed__5() { -_start: +else { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabAttr___boxed), 4, 0); -return x_1; +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_17, 1); +lean_inc(x_23); +lean_dec(x_17); +lean_inc(x_16); +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_16); +lean_ctor_set(x_24, 1, x_16); +x_25 = l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabInitialize___spec__4(x_1, x_24, x_4, x_5, x_23); +lean_dec(x_4); +return x_25; } } -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabAttr__1(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; -x_2 = l___regBuiltin_Lean_Elab_Command_elabDeclaration__1___closed__3; -x_3 = l___regBuiltin_Lean_Elab_Command_elabAttr__1___closed__2; -x_4 = l___regBuiltin_Lean_Elab_Command_elabAttr__1___closed__4; -x_5 = l___regBuiltin_Lean_Elab_Command_elabAttr__1___closed__5; -x_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_elabAttr_declRange__1___closed__1() { -_start: +uint8_t x_26; +x_26 = !lean_is_exclusive(x_17); +if (x_26 == 0) { -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(36u); -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_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_27 = lean_ctor_get(x_17, 1); +x_28 = lean_ctor_get(x_17, 0); +lean_dec(x_28); +x_29 = lean_ctor_get(x_18, 0); +lean_inc(x_29); +lean_dec(x_18); +lean_ctor_set(x_17, 1, x_29); +lean_ctor_set(x_17, 0, x_16); +x_30 = l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabInitialize___spec__4(x_1, x_17, x_4, x_5, x_27); +lean_dec(x_4); +return x_30; } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1___closed__2() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(383u); -x_2 = lean_unsigned_to_nat(39u); -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_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_31 = lean_ctor_get(x_17, 1); +lean_inc(x_31); +lean_dec(x_17); +x_32 = lean_ctor_get(x_18, 0); +lean_inc(x_32); +lean_dec(x_18); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_16); +lean_ctor_set(x_33, 1, x_32); +x_34 = l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabInitialize___spec__4(x_1, x_33, x_4, x_5, x_31); +lean_dec(x_4); +return x_34; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1___closed__1; -x_2 = lean_unsigned_to_nat(36u); -x_3 = l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1___closed__2; -x_4 = lean_unsigned_to_nat(39u); -x_5 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_5, 0, x_1); -lean_ctor_set(x_5, 1, x_2); -lean_ctor_set(x_5, 2, x_3); -lean_ctor_set(x_5, 3, x_4); -return x_5; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1___closed__4() { +} +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Command_elabInitialize___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_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(351u); -x_2 = lean_unsigned_to_nat(40u); -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; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_8 = lean_box(0); +lean_inc(x_1); +x_9 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_9, 0, x_1); +lean_ctor_set(x_9, 1, x_8); +x_10 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_10, 0, x_2); +lean_ctor_set(x_10, 1, x_9); +x_11 = lean_array_mk(x_10); +x_12 = lean_box(2); +x_13 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; +x_14 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_14, 0, x_12); +lean_ctor_set(x_14, 1, x_13); +lean_ctor_set(x_14, 2, x_11); +x_15 = l_Lean_Elab_getDeclarationSelectionRef(x_1); +x_16 = l_Lean_Elab_addDeclarationRangesFromSyntax___at_Lean_Elab_Command_elabInitialize___spec__2(x_3, x_14, x_15, x_5, x_6, x_7); +lean_dec(x_15); +lean_dec(x_14); +return x_16; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1___closed__5() { +static lean_object* _init_l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Command_elabInitialize___spec__1___closed__1() { _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(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; +x_1 = lean_mk_string_unchecked("example", 7, 7); +return x_1; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1___closed__6() { +static lean_object* _init_l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Command_elabInitialize___spec__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1___closed__4; -x_2 = lean_unsigned_to_nat(40u); -x_3 = l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1___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); +x_1 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__1; +x_2 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__2; +x_3 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__3; +x_4 = l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Command_elabInitialize___spec__1___closed__1; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1___closed__7() { +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Command_elabInitialize___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_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1___closed__3; -x_2 = l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__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; -} +lean_object* x_7; lean_object* x_8; uint8_t x_9; +lean_inc(x_3); +x_7 = l_Lean_Syntax_getKind(x_3); +x_8 = l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Command_elabInitialize___spec__1___closed__2; +x_9 = lean_name_eq(x_7, x_8); +lean_dec(x_7); +if (x_9 == 0) +{ +lean_object* x_10; lean_object* x_11; +x_10 = lean_box(0); +x_11 = l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Command_elabInitialize___spec__1___lambda__1(x_3, x_2, x_1, x_10, x_4, x_5, x_6); +return x_11; } -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1(lean_object* x_1) { -_start: +else { -lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_2 = l___regBuiltin_Lean_Elab_Command_elabAttr__1___closed__4; -x_3 = l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1___closed__7; -x_4 = l_Lean_addBuiltinDeclarationRanges(x_2, x_3, x_1); -return x_4; +lean_object* x_12; lean_object* x_13; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_12 = lean_box(0); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_6); +return x_13; +} } } static lean_object* _init_l_Lean_Elab_Command_elabInitialize___lambda__1___closed__1() { @@ -11400,23 +9175,31 @@ static lean_object* _init_l_Lean_Elab_Command_elabInitialize___lambda__1___close _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("do", 2, 2); +x_1 = lean_mk_string_unchecked(":=", 2, 2); return x_1; } } static lean_object* _init_l_Lean_Elab_Command_elabInitialize___lambda__1___closed__44() { _start: { +lean_object* x_1; +x_1 = lean_mk_string_unchecked("do", 2, 2); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabInitialize___lambda__1___closed__45() { +_start: +{ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__1; x_2 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__2; x_3 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__3; -x_4 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__43; +x_4 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__44; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Elab_Command_elabInitialize___lambda__1___closed__45() { +static lean_object* _init_l_Lean_Elab_Command_elabInitialize___lambda__1___closed__46() { _start: { lean_object* x_1; @@ -11424,7 +9207,7 @@ x_1 = lean_mk_string_unchecked("Termination", 11, 11); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_elabInitialize___lambda__1___closed__46() { +static lean_object* _init_l_Lean_Elab_Command_elabInitialize___lambda__1___closed__47() { _start: { lean_object* x_1; @@ -11432,19 +9215,19 @@ x_1 = lean_mk_string_unchecked("suffix", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_elabInitialize___lambda__1___closed__47() { +static lean_object* _init_l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__1; x_2 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__2; -x_3 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__45; -x_4 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__46; +x_3 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__46; +x_4 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__47; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48() { +static lean_object* _init_l_Lean_Elab_Command_elabInitialize___lambda__1___closed__49() { _start: { lean_object* x_1; lean_object* x_2; @@ -11669,20 +9452,20 @@ x_91 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__21; lean_inc(x_53); lean_inc(x_41); x_92 = l_Lean_Syntax_node2(x_41, x_91, x_53, x_90); -x_93 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1; +x_93 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__43; lean_inc(x_41); x_94 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_94, 0, x_41); lean_ctor_set(x_94, 1, x_93); -x_95 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__43; +x_95 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__44; lean_inc(x_41); x_96 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_96, 0, x_41); lean_ctor_set(x_96, 1, x_95); -x_97 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__44; +x_97 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__45; lean_inc(x_41); x_98 = l_Lean_Syntax_node2(x_41, x_97, x_96, x_3); -x_99 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__47; +x_99 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48; lean_inc_n(x_53, 2); lean_inc(x_41); x_100 = l_Lean_Syntax_node2(x_41, x_99, x_53, x_53); @@ -11697,7 +9480,7 @@ x_104 = l_Lean_Syntax_node5(x_41, x_103, x_36, x_72, x_92, x_102, x_53); if (lean_obj_tag(x_6) == 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; -x_105 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48; +x_105 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__49; lean_inc(x_41); x_106 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_106, 0, x_41); @@ -11839,20 +9622,20 @@ x_163 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__21; lean_inc(x_125); lean_inc(x_41); x_164 = l_Lean_Syntax_node2(x_41, x_163, x_125, x_162); -x_165 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1; +x_165 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__43; lean_inc(x_41); x_166 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_166, 0, x_41); lean_ctor_set(x_166, 1, x_165); -x_167 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__43; +x_167 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__44; lean_inc(x_41); x_168 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_168, 0, x_41); lean_ctor_set(x_168, 1, x_167); -x_169 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__44; +x_169 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__45; lean_inc(x_41); x_170 = l_Lean_Syntax_node2(x_41, x_169, x_168, x_3); -x_171 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__47; +x_171 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48; lean_inc_n(x_125, 2); lean_inc(x_41); x_172 = l_Lean_Syntax_node2(x_41, x_171, x_125, x_125); @@ -11867,7 +9650,7 @@ x_176 = l_Lean_Syntax_node5(x_41, x_175, x_36, x_144, x_164, x_174, x_125); if (lean_obj_tag(x_6) == 0) { 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_177 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48; +x_177 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__49; lean_inc(x_41); x_178 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_178, 0, x_41); @@ -12028,20 +9811,20 @@ x_240 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__21; lean_inc(x_201); lean_inc(x_41); x_241 = l_Lean_Syntax_node2(x_41, x_240, x_201, x_239); -x_242 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1; +x_242 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__43; lean_inc(x_41); x_243 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_243, 0, x_41); lean_ctor_set(x_243, 1, x_242); -x_244 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__43; +x_244 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__44; lean_inc(x_41); x_245 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_245, 0, x_41); lean_ctor_set(x_245, 1, x_244); -x_246 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__44; +x_246 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__45; lean_inc(x_41); x_247 = l_Lean_Syntax_node2(x_41, x_246, x_245, x_3); -x_248 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__47; +x_248 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48; lean_inc_n(x_201, 2); lean_inc(x_41); x_249 = l_Lean_Syntax_node2(x_41, x_248, x_201, x_201); @@ -12056,7 +9839,7 @@ x_253 = l_Lean_Syntax_node5(x_41, x_252, x_36, x_221, x_241, x_251, x_201); if (lean_obj_tag(x_6) == 0) { lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; -x_254 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48; +x_254 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__49; lean_inc(x_41); x_255 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_255, 0, x_41); @@ -12238,20 +10021,20 @@ x_324 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__21; lean_inc(x_284); lean_inc(x_271); x_325 = l_Lean_Syntax_node2(x_271, x_324, x_284, x_323); -x_326 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1; +x_326 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__43; lean_inc(x_271); x_327 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_327, 0, x_271); lean_ctor_set(x_327, 1, x_326); -x_328 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__43; +x_328 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__44; lean_inc(x_271); x_329 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_329, 0, x_271); lean_ctor_set(x_329, 1, x_328); -x_330 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__44; +x_330 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__45; lean_inc(x_271); x_331 = l_Lean_Syntax_node2(x_271, x_330, x_329, x_3); -x_332 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__47; +x_332 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48; lean_inc_n(x_284, 2); lean_inc(x_271); x_333 = l_Lean_Syntax_node2(x_271, x_332, x_284, x_284); @@ -12266,7 +10049,7 @@ x_337 = l_Lean_Syntax_node5(x_271, x_336, x_298, x_305, x_325, x_335, x_284); if (lean_obj_tag(x_6) == 0) { lean_object* x_338; lean_object* x_339; lean_object* x_340; lean_object* x_341; lean_object* x_342; lean_object* x_343; -x_338 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48; +x_338 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__49; lean_inc(x_271); x_339 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_339, 0, x_271); @@ -12361,532 +10144,522 @@ return x_5; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInitialize___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_11; uint8_t x_12; +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_11 = lean_unsigned_to_nat(0u); +x_12 = l_Lean_Syntax_getArg(x_1, x_11); +x_13 = lean_unsigned_to_nat(1u); +x_14 = l_Lean_Syntax_getArg(x_1, x_13); lean_inc(x_8); -lean_inc(x_1); lean_inc(x_6); -x_11 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1(x_6, x_1, x_8, x_9, x_10); -x_12 = !lean_is_exclusive(x_11); -if (x_12 == 0) -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; -x_13 = lean_ctor_get(x_11, 1); -x_14 = lean_ctor_get(x_11, 0); -lean_dec(x_14); -x_15 = l_Lean_Elab_Command_getRef(x_8, x_9, x_13); +x_15 = l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Command_elabInitialize___spec__1(x_6, x_12, x_14, x_8, x_9, x_10); x_16 = !lean_is_exclusive(x_15); if (x_16 == 0) { -lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; -x_17 = lean_ctor_get(x_15, 0); -x_18 = lean_ctor_get(x_15, 1); -x_19 = 0; -x_20 = l_Lean_SourceInfo_fromRef(x_17, x_19); -lean_dec(x_17); -x_21 = l_Lean_Elab_Command_getCurrMacroScope(x_8, x_9, x_18); -x_22 = !lean_is_exclusive(x_21); -if (x_22 == 0) +lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; +x_17 = lean_ctor_get(x_15, 1); +x_18 = lean_ctor_get(x_15, 0); +lean_dec(x_18); +x_19 = l_Lean_Elab_Command_getRef(x_8, x_9, x_17); +x_20 = !lean_is_exclusive(x_19); +if (x_20 == 0) { -lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; -x_23 = lean_ctor_get(x_21, 0); -x_24 = lean_ctor_get(x_21, 1); -x_25 = l_Lean_Elab_Command_getMainModule___rarg(x_9, x_24); +lean_object* x_21; lean_object* x_22; uint8_t x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; +x_21 = lean_ctor_get(x_19, 0); +x_22 = lean_ctor_get(x_19, 1); +x_23 = 0; +x_24 = l_Lean_SourceInfo_fromRef(x_21, x_23); +lean_dec(x_21); +x_25 = l_Lean_Elab_Command_getCurrMacroScope(x_8, x_9, x_22); x_26 = !lean_is_exclusive(x_25); if (x_26 == 0) { -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; +lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; x_27 = lean_ctor_get(x_25, 0); x_28 = lean_ctor_get(x_25, 1); -x_29 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; -x_30 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; -lean_inc(x_20); -x_31 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_31, 0, x_20); -lean_ctor_set(x_31, 1, x_29); -lean_ctor_set(x_31, 2, x_30); -x_32 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__14; -lean_inc(x_20); -lean_ctor_set_tag(x_25, 2); -lean_ctor_set(x_25, 1, x_32); -lean_ctor_set(x_25, 0, x_20); -x_33 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__19; -lean_inc(x_23); +x_29 = l_Lean_Elab_Command_getMainModule___rarg(x_9, x_28); +x_30 = !lean_is_exclusive(x_29); +if (x_30 == 0) +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; +x_31 = lean_ctor_get(x_29, 0); +x_32 = lean_ctor_get(x_29, 1); +x_33 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; +x_34 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; +lean_inc(x_24); +x_35 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_35, 0, x_24); +lean_ctor_set(x_35, 1, x_33); +lean_ctor_set(x_35, 2, x_34); +x_36 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__14; +lean_inc(x_24); +lean_ctor_set_tag(x_29, 2); +lean_ctor_set(x_29, 1, x_36); +lean_ctor_set(x_29, 0, x_24); +x_37 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__19; lean_inc(x_27); -x_34 = l_Lean_addMacroScope(x_27, x_33, x_23); -x_35 = lean_box(0); -x_36 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__18; -lean_inc(x_20); -x_37 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_37, 0, x_20); -lean_ctor_set(x_37, 1, x_36); -lean_ctor_set(x_37, 2, x_34); -lean_ctor_set(x_37, 3, x_35); -x_38 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__16; -lean_inc(x_31); -lean_inc(x_20); -x_39 = l_Lean_Syntax_node2(x_20, x_38, x_37, x_31); -x_40 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__24; -lean_inc(x_20); -lean_ctor_set_tag(x_21, 2); -lean_ctor_set(x_21, 1, x_40); -lean_ctor_set(x_21, 0, x_20); -x_41 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__29; -x_42 = l_Lean_addMacroScope(x_27, x_41, x_23); -x_43 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__28; -x_44 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__33; -lean_inc(x_20); -x_45 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_45, 0, x_20); -lean_ctor_set(x_45, 1, x_43); -lean_ctor_set(x_45, 2, x_42); -lean_ctor_set(x_45, 3, x_44); -lean_inc(x_20); -x_46 = l_Lean_Syntax_node1(x_20, x_29, x_2); -x_47 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__26; -lean_inc(x_20); -x_48 = l_Lean_Syntax_node2(x_20, x_47, x_45, x_46); -x_49 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__23; -lean_inc(x_20); -x_50 = l_Lean_Syntax_node2(x_20, x_49, x_21, x_48); -lean_inc(x_20); -x_51 = l_Lean_Syntax_node1(x_20, x_29, x_50); -x_52 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__21; -lean_inc(x_31); -lean_inc(x_20); -x_53 = l_Lean_Syntax_node2(x_20, x_52, x_31, x_51); -x_54 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1; -lean_inc(x_20); -lean_ctor_set_tag(x_15, 2); -lean_ctor_set(x_15, 1, x_54); -lean_ctor_set(x_15, 0, x_20); -x_55 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__3; -lean_inc(x_20); -lean_ctor_set_tag(x_11, 2); -lean_ctor_set(x_11, 1, x_55); -lean_ctor_set(x_11, 0, x_20); -x_56 = lean_mk_syntax_ident(x_6); -x_57 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__43; -lean_inc(x_20); -x_58 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_58, 0, x_20); -lean_ctor_set(x_58, 1, x_57); -x_59 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__44; -lean_inc(x_20); -x_60 = l_Lean_Syntax_node2(x_20, x_59, x_58, x_3); -x_61 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__2; -lean_inc(x_31); -lean_inc(x_20); -x_62 = l_Lean_Syntax_node4(x_20, x_61, x_11, x_31, x_56, x_60); -x_63 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__47; -lean_inc_n(x_31, 2); -lean_inc(x_20); -x_64 = l_Lean_Syntax_node2(x_20, x_63, x_31, x_31); -x_65 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__42; lean_inc(x_31); -lean_inc(x_20); -x_66 = l_Lean_Syntax_node4(x_20, x_65, x_15, x_62, x_64, x_31); -x_67 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__9; -lean_inc(x_31); -lean_inc(x_20); -x_68 = l_Lean_Syntax_node5(x_20, x_67, x_25, x_39, x_53, x_66, x_31); -if (lean_obj_tag(x_4) == 0) -{ -lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; -x_69 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48; -lean_inc(x_20); -x_70 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_70, 0, x_20); -lean_ctor_set(x_70, 1, x_29); -lean_ctor_set(x_70, 2, x_69); -lean_inc_n(x_31, 4); -lean_inc(x_20); -x_71 = l_Lean_Syntax_node6(x_20, x_5, x_31, x_31, x_31, x_31, x_70, x_31); -x_72 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; -lean_inc(x_20); -x_73 = l_Lean_Syntax_node2(x_20, x_72, x_71, x_68); -x_74 = l_Lean_Syntax_node2(x_20, x_29, x_73, x_1); -x_75 = l_Lean_Elab_Command_elabCommand(x_74, x_8, x_9, x_28); -return x_75; -} -else -{ -lean_object* x_76; uint8_t x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; -x_76 = lean_ctor_get(x_4, 0); -x_77 = 1; -x_78 = l_Lean_SourceInfo_fromRef(x_76, x_77); -x_79 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__4; -x_80 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_80, 0, x_78); -lean_ctor_set(x_80, 1, x_79); -x_81 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__5; -lean_inc(x_20); -x_82 = l_Lean_Syntax_node1(x_20, x_81, x_80); -x_83 = l_Array_mkArray1___rarg(x_82); -x_84 = l_Array_append___rarg(x_30, x_83); -lean_dec(x_83); -lean_inc(x_20); -x_85 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_85, 0, x_20); -lean_ctor_set(x_85, 1, x_29); -lean_ctor_set(x_85, 2, x_84); -lean_inc_n(x_31, 4); -lean_inc(x_20); -x_86 = l_Lean_Syntax_node6(x_20, x_5, x_31, x_31, x_31, x_31, x_85, x_31); -x_87 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; -lean_inc(x_20); -x_88 = l_Lean_Syntax_node2(x_20, x_87, x_86, x_68); -x_89 = l_Lean_Syntax_node2(x_20, x_29, x_88, x_1); -x_90 = l_Lean_Elab_Command_elabCommand(x_89, x_8, x_9, x_28); -return x_90; -} -} -else -{ -lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; -x_91 = lean_ctor_get(x_25, 0); -x_92 = lean_ctor_get(x_25, 1); -lean_inc(x_92); -lean_inc(x_91); -lean_dec(x_25); -x_93 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; -x_94 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; -lean_inc(x_20); -x_95 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_95, 0, x_20); -lean_ctor_set(x_95, 1, x_93); -lean_ctor_set(x_95, 2, x_94); -x_96 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__14; -lean_inc(x_20); -x_97 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_97, 0, x_20); -lean_ctor_set(x_97, 1, x_96); -x_98 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__19; -lean_inc(x_23); -lean_inc(x_91); -x_99 = l_Lean_addMacroScope(x_91, x_98, x_23); -x_100 = lean_box(0); -x_101 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__18; -lean_inc(x_20); -x_102 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_102, 0, x_20); -lean_ctor_set(x_102, 1, x_101); -lean_ctor_set(x_102, 2, x_99); -lean_ctor_set(x_102, 3, x_100); -x_103 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__16; -lean_inc(x_95); -lean_inc(x_20); -x_104 = l_Lean_Syntax_node2(x_20, x_103, x_102, x_95); -x_105 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__24; -lean_inc(x_20); -lean_ctor_set_tag(x_21, 2); -lean_ctor_set(x_21, 1, x_105); -lean_ctor_set(x_21, 0, x_20); -x_106 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__29; -x_107 = l_Lean_addMacroScope(x_91, x_106, x_23); -x_108 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__28; -x_109 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__33; -lean_inc(x_20); -x_110 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_110, 0, x_20); -lean_ctor_set(x_110, 1, x_108); -lean_ctor_set(x_110, 2, x_107); -lean_ctor_set(x_110, 3, x_109); -lean_inc(x_20); -x_111 = l_Lean_Syntax_node1(x_20, x_93, x_2); -x_112 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__26; -lean_inc(x_20); -x_113 = l_Lean_Syntax_node2(x_20, x_112, x_110, x_111); -x_114 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__23; -lean_inc(x_20); -x_115 = l_Lean_Syntax_node2(x_20, x_114, x_21, x_113); -lean_inc(x_20); -x_116 = l_Lean_Syntax_node1(x_20, x_93, x_115); -x_117 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__21; -lean_inc(x_95); -lean_inc(x_20); -x_118 = l_Lean_Syntax_node2(x_20, x_117, x_95, x_116); -x_119 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1; -lean_inc(x_20); +x_38 = l_Lean_addMacroScope(x_31, x_37, x_27); +x_39 = lean_box(0); +x_40 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__18; +lean_inc(x_24); +x_41 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_41, 0, x_24); +lean_ctor_set(x_41, 1, x_40); +lean_ctor_set(x_41, 2, x_38); +lean_ctor_set(x_41, 3, x_39); +x_42 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__16; +lean_inc(x_35); +lean_inc(x_24); +x_43 = l_Lean_Syntax_node2(x_24, x_42, x_41, x_35); +x_44 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__24; +lean_inc(x_24); +lean_ctor_set_tag(x_25, 2); +lean_ctor_set(x_25, 1, x_44); +lean_ctor_set(x_25, 0, x_24); +x_45 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__29; +x_46 = l_Lean_addMacroScope(x_31, x_45, x_27); +x_47 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__28; +x_48 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__33; +lean_inc(x_24); +x_49 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_49, 0, x_24); +lean_ctor_set(x_49, 1, x_47); +lean_ctor_set(x_49, 2, x_46); +lean_ctor_set(x_49, 3, x_48); +lean_inc(x_24); +x_50 = l_Lean_Syntax_node1(x_24, x_33, x_2); +x_51 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__26; +lean_inc(x_24); +x_52 = l_Lean_Syntax_node2(x_24, x_51, x_49, x_50); +x_53 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__23; +lean_inc(x_24); +x_54 = l_Lean_Syntax_node2(x_24, x_53, x_25, x_52); +lean_inc(x_24); +x_55 = l_Lean_Syntax_node1(x_24, x_33, x_54); +x_56 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__21; +lean_inc(x_35); +lean_inc(x_24); +x_57 = l_Lean_Syntax_node2(x_24, x_56, x_35, x_55); +x_58 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__43; +lean_inc(x_24); +lean_ctor_set_tag(x_19, 2); +lean_ctor_set(x_19, 1, x_58); +lean_ctor_set(x_19, 0, x_24); +x_59 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__3; +lean_inc(x_24); lean_ctor_set_tag(x_15, 2); -lean_ctor_set(x_15, 1, x_119); -lean_ctor_set(x_15, 0, x_20); -x_120 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__3; -lean_inc(x_20); -lean_ctor_set_tag(x_11, 2); -lean_ctor_set(x_11, 1, x_120); -lean_ctor_set(x_11, 0, x_20); -x_121 = lean_mk_syntax_ident(x_6); -x_122 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__43; -lean_inc(x_20); -x_123 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_123, 0, x_20); -lean_ctor_set(x_123, 1, x_122); -x_124 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__44; -lean_inc(x_20); -x_125 = l_Lean_Syntax_node2(x_20, x_124, x_123, x_3); -x_126 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__2; -lean_inc(x_95); -lean_inc(x_20); -x_127 = l_Lean_Syntax_node4(x_20, x_126, x_11, x_95, x_121, x_125); -x_128 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__47; -lean_inc_n(x_95, 2); -lean_inc(x_20); -x_129 = l_Lean_Syntax_node2(x_20, x_128, x_95, x_95); -x_130 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__42; +lean_ctor_set(x_15, 1, x_59); +lean_ctor_set(x_15, 0, x_24); +x_60 = lean_mk_syntax_ident(x_6); +x_61 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__44; +lean_inc(x_24); +x_62 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_62, 0, x_24); +lean_ctor_set(x_62, 1, x_61); +x_63 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__45; +lean_inc(x_24); +x_64 = l_Lean_Syntax_node2(x_24, x_63, x_62, x_3); +x_65 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__2; +lean_inc(x_35); +lean_inc(x_24); +x_66 = l_Lean_Syntax_node4(x_24, x_65, x_15, x_35, x_60, x_64); +x_67 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48; +lean_inc_n(x_35, 2); +lean_inc(x_24); +x_68 = l_Lean_Syntax_node2(x_24, x_67, x_35, x_35); +x_69 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__42; +lean_inc(x_35); +lean_inc(x_24); +x_70 = l_Lean_Syntax_node4(x_24, x_69, x_19, x_66, x_68, x_35); +x_71 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__9; +lean_inc(x_35); +lean_inc(x_24); +x_72 = l_Lean_Syntax_node5(x_24, x_71, x_29, x_43, x_57, x_70, x_35); +if (lean_obj_tag(x_4) == 0) +{ +lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; +x_73 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__49; +lean_inc(x_24); +x_74 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_74, 0, x_24); +lean_ctor_set(x_74, 1, x_33); +lean_ctor_set(x_74, 2, x_73); +lean_inc_n(x_35, 4); +lean_inc(x_24); +x_75 = l_Lean_Syntax_node6(x_24, x_5, x_35, x_35, x_35, x_35, x_74, x_35); +x_76 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; +lean_inc(x_24); +x_77 = l_Lean_Syntax_node2(x_24, x_76, x_75, x_72); +x_78 = l_Lean_Syntax_node2(x_24, x_33, x_77, x_1); +x_79 = l_Lean_Elab_Command_elabCommand(x_78, x_8, x_9, x_32); +return x_79; +} +else +{ +lean_object* x_80; uint8_t x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; +x_80 = lean_ctor_get(x_4, 0); +x_81 = 1; +x_82 = l_Lean_SourceInfo_fromRef(x_80, x_81); +x_83 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__4; +x_84 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_84, 0, x_82); +lean_ctor_set(x_84, 1, x_83); +x_85 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__5; +lean_inc(x_24); +x_86 = l_Lean_Syntax_node1(x_24, x_85, x_84); +x_87 = l_Array_mkArray1___rarg(x_86); +x_88 = l_Array_append___rarg(x_34, x_87); +lean_dec(x_87); +lean_inc(x_24); +x_89 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_89, 0, x_24); +lean_ctor_set(x_89, 1, x_33); +lean_ctor_set(x_89, 2, x_88); +lean_inc_n(x_35, 4); +lean_inc(x_24); +x_90 = l_Lean_Syntax_node6(x_24, x_5, x_35, x_35, x_35, x_35, x_89, x_35); +x_91 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; +lean_inc(x_24); +x_92 = l_Lean_Syntax_node2(x_24, x_91, x_90, x_72); +x_93 = l_Lean_Syntax_node2(x_24, x_33, x_92, x_1); +x_94 = l_Lean_Elab_Command_elabCommand(x_93, x_8, x_9, x_32); +return x_94; +} +} +else +{ +lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; +x_95 = lean_ctor_get(x_29, 0); +x_96 = lean_ctor_get(x_29, 1); +lean_inc(x_96); lean_inc(x_95); -lean_inc(x_20); -x_131 = l_Lean_Syntax_node4(x_20, x_130, x_15, x_127, x_129, x_95); -x_132 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__9; +lean_dec(x_29); +x_97 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; +x_98 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; +lean_inc(x_24); +x_99 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_99, 0, x_24); +lean_ctor_set(x_99, 1, x_97); +lean_ctor_set(x_99, 2, x_98); +x_100 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__14; +lean_inc(x_24); +x_101 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_101, 0, x_24); +lean_ctor_set(x_101, 1, x_100); +x_102 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__19; +lean_inc(x_27); lean_inc(x_95); -lean_inc(x_20); -x_133 = l_Lean_Syntax_node5(x_20, x_132, x_97, x_104, x_118, x_131, x_95); +x_103 = l_Lean_addMacroScope(x_95, x_102, x_27); +x_104 = lean_box(0); +x_105 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__18; +lean_inc(x_24); +x_106 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_106, 0, x_24); +lean_ctor_set(x_106, 1, x_105); +lean_ctor_set(x_106, 2, x_103); +lean_ctor_set(x_106, 3, x_104); +x_107 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__16; +lean_inc(x_99); +lean_inc(x_24); +x_108 = l_Lean_Syntax_node2(x_24, x_107, x_106, x_99); +x_109 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__24; +lean_inc(x_24); +lean_ctor_set_tag(x_25, 2); +lean_ctor_set(x_25, 1, x_109); +lean_ctor_set(x_25, 0, x_24); +x_110 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__29; +x_111 = l_Lean_addMacroScope(x_95, x_110, x_27); +x_112 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__28; +x_113 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__33; +lean_inc(x_24); +x_114 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_114, 0, x_24); +lean_ctor_set(x_114, 1, x_112); +lean_ctor_set(x_114, 2, x_111); +lean_ctor_set(x_114, 3, x_113); +lean_inc(x_24); +x_115 = l_Lean_Syntax_node1(x_24, x_97, x_2); +x_116 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__26; +lean_inc(x_24); +x_117 = l_Lean_Syntax_node2(x_24, x_116, x_114, x_115); +x_118 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__23; +lean_inc(x_24); +x_119 = l_Lean_Syntax_node2(x_24, x_118, x_25, x_117); +lean_inc(x_24); +x_120 = l_Lean_Syntax_node1(x_24, x_97, x_119); +x_121 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__21; +lean_inc(x_99); +lean_inc(x_24); +x_122 = l_Lean_Syntax_node2(x_24, x_121, x_99, x_120); +x_123 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__43; +lean_inc(x_24); +lean_ctor_set_tag(x_19, 2); +lean_ctor_set(x_19, 1, x_123); +lean_ctor_set(x_19, 0, x_24); +x_124 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__3; +lean_inc(x_24); +lean_ctor_set_tag(x_15, 2); +lean_ctor_set(x_15, 1, x_124); +lean_ctor_set(x_15, 0, x_24); +x_125 = lean_mk_syntax_ident(x_6); +x_126 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__44; +lean_inc(x_24); +x_127 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_127, 0, x_24); +lean_ctor_set(x_127, 1, x_126); +x_128 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__45; +lean_inc(x_24); +x_129 = l_Lean_Syntax_node2(x_24, x_128, x_127, x_3); +x_130 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__2; +lean_inc(x_99); +lean_inc(x_24); +x_131 = l_Lean_Syntax_node4(x_24, x_130, x_15, x_99, x_125, x_129); +x_132 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48; +lean_inc_n(x_99, 2); +lean_inc(x_24); +x_133 = l_Lean_Syntax_node2(x_24, x_132, x_99, x_99); +x_134 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__42; +lean_inc(x_99); +lean_inc(x_24); +x_135 = l_Lean_Syntax_node4(x_24, x_134, x_19, x_131, x_133, x_99); +x_136 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__9; +lean_inc(x_99); +lean_inc(x_24); +x_137 = l_Lean_Syntax_node5(x_24, x_136, x_101, x_108, x_122, x_135, x_99); if (lean_obj_tag(x_4) == 0) { -lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; -x_134 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48; -lean_inc(x_20); -x_135 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_135, 0, x_20); -lean_ctor_set(x_135, 1, x_93); -lean_ctor_set(x_135, 2, x_134); -lean_inc_n(x_95, 4); -lean_inc(x_20); -x_136 = l_Lean_Syntax_node6(x_20, x_5, x_95, x_95, x_95, x_95, x_135, x_95); -x_137 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; -lean_inc(x_20); -x_138 = l_Lean_Syntax_node2(x_20, x_137, x_136, x_133); -x_139 = l_Lean_Syntax_node2(x_20, x_93, x_138, x_1); -x_140 = l_Lean_Elab_Command_elabCommand(x_139, x_8, x_9, x_92); -return x_140; +lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; +x_138 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__49; +lean_inc(x_24); +x_139 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_139, 0, x_24); +lean_ctor_set(x_139, 1, x_97); +lean_ctor_set(x_139, 2, x_138); +lean_inc_n(x_99, 4); +lean_inc(x_24); +x_140 = l_Lean_Syntax_node6(x_24, x_5, x_99, x_99, x_99, x_99, x_139, x_99); +x_141 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; +lean_inc(x_24); +x_142 = l_Lean_Syntax_node2(x_24, x_141, x_140, x_137); +x_143 = l_Lean_Syntax_node2(x_24, x_97, x_142, x_1); +x_144 = l_Lean_Elab_Command_elabCommand(x_143, x_8, x_9, x_96); +return x_144; } else { -lean_object* x_141; uint8_t x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; -x_141 = lean_ctor_get(x_4, 0); -x_142 = 1; -x_143 = l_Lean_SourceInfo_fromRef(x_141, x_142); -x_144 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__4; -x_145 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_145, 0, x_143); -lean_ctor_set(x_145, 1, x_144); -x_146 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__5; -lean_inc(x_20); -x_147 = l_Lean_Syntax_node1(x_20, x_146, x_145); -x_148 = l_Array_mkArray1___rarg(x_147); -x_149 = l_Array_append___rarg(x_94, x_148); -lean_dec(x_148); -lean_inc(x_20); -x_150 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_150, 0, x_20); -lean_ctor_set(x_150, 1, x_93); -lean_ctor_set(x_150, 2, x_149); -lean_inc_n(x_95, 4); -lean_inc(x_20); -x_151 = l_Lean_Syntax_node6(x_20, x_5, x_95, x_95, x_95, x_95, x_150, x_95); -x_152 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; -lean_inc(x_20); -x_153 = l_Lean_Syntax_node2(x_20, x_152, x_151, x_133); -x_154 = l_Lean_Syntax_node2(x_20, x_93, x_153, x_1); -x_155 = l_Lean_Elab_Command_elabCommand(x_154, x_8, x_9, x_92); -return x_155; +lean_object* x_145; uint8_t x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; +x_145 = lean_ctor_get(x_4, 0); +x_146 = 1; +x_147 = l_Lean_SourceInfo_fromRef(x_145, x_146); +x_148 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__4; +x_149 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_149, 0, x_147); +lean_ctor_set(x_149, 1, x_148); +x_150 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__5; +lean_inc(x_24); +x_151 = l_Lean_Syntax_node1(x_24, x_150, x_149); +x_152 = l_Array_mkArray1___rarg(x_151); +x_153 = l_Array_append___rarg(x_98, x_152); +lean_dec(x_152); +lean_inc(x_24); +x_154 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_154, 0, x_24); +lean_ctor_set(x_154, 1, x_97); +lean_ctor_set(x_154, 2, x_153); +lean_inc_n(x_99, 4); +lean_inc(x_24); +x_155 = l_Lean_Syntax_node6(x_24, x_5, x_99, x_99, x_99, x_99, x_154, x_99); +x_156 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; +lean_inc(x_24); +x_157 = l_Lean_Syntax_node2(x_24, x_156, x_155, x_137); +x_158 = l_Lean_Syntax_node2(x_24, x_97, x_157, x_1); +x_159 = l_Lean_Elab_Command_elabCommand(x_158, x_8, x_9, x_96); +return x_159; } } } else { -lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; -x_156 = lean_ctor_get(x_21, 0); -x_157 = lean_ctor_get(x_21, 1); -lean_inc(x_157); -lean_inc(x_156); -lean_dec(x_21); -x_158 = l_Lean_Elab_Command_getMainModule___rarg(x_9, x_157); -x_159 = lean_ctor_get(x_158, 0); -lean_inc(x_159); -x_160 = lean_ctor_get(x_158, 1); +lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; +x_160 = lean_ctor_get(x_25, 0); +x_161 = lean_ctor_get(x_25, 1); +lean_inc(x_161); lean_inc(x_160); -if (lean_is_exclusive(x_158)) { - lean_ctor_release(x_158, 0); - lean_ctor_release(x_158, 1); - x_161 = x_158; +lean_dec(x_25); +x_162 = l_Lean_Elab_Command_getMainModule___rarg(x_9, x_161); +x_163 = lean_ctor_get(x_162, 0); +lean_inc(x_163); +x_164 = lean_ctor_get(x_162, 1); +lean_inc(x_164); +if (lean_is_exclusive(x_162)) { + lean_ctor_release(x_162, 0); + lean_ctor_release(x_162, 1); + x_165 = x_162; } else { - lean_dec_ref(x_158); - x_161 = lean_box(0); + lean_dec_ref(x_162); + x_165 = lean_box(0); } -x_162 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; -x_163 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; -lean_inc(x_20); -x_164 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_164, 0, x_20); -lean_ctor_set(x_164, 1, x_162); -lean_ctor_set(x_164, 2, x_163); -x_165 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__14; -lean_inc(x_20); -if (lean_is_scalar(x_161)) { - x_166 = lean_alloc_ctor(2, 2, 0); +x_166 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; +x_167 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; +lean_inc(x_24); +x_168 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_168, 0, x_24); +lean_ctor_set(x_168, 1, x_166); +lean_ctor_set(x_168, 2, x_167); +x_169 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__14; +lean_inc(x_24); +if (lean_is_scalar(x_165)) { + x_170 = lean_alloc_ctor(2, 2, 0); } else { - x_166 = x_161; - lean_ctor_set_tag(x_166, 2); + x_170 = x_165; + lean_ctor_set_tag(x_170, 2); } -lean_ctor_set(x_166, 0, x_20); -lean_ctor_set(x_166, 1, x_165); -x_167 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__19; -lean_inc(x_156); -lean_inc(x_159); -x_168 = l_Lean_addMacroScope(x_159, x_167, x_156); -x_169 = lean_box(0); -x_170 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__18; -lean_inc(x_20); -x_171 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_171, 0, x_20); -lean_ctor_set(x_171, 1, x_170); -lean_ctor_set(x_171, 2, x_168); -lean_ctor_set(x_171, 3, x_169); -x_172 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__16; -lean_inc(x_164); -lean_inc(x_20); -x_173 = l_Lean_Syntax_node2(x_20, x_172, x_171, x_164); -x_174 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__24; -lean_inc(x_20); -x_175 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_175, 0, x_20); +lean_ctor_set(x_170, 0, x_24); +lean_ctor_set(x_170, 1, x_169); +x_171 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__19; +lean_inc(x_160); +lean_inc(x_163); +x_172 = l_Lean_addMacroScope(x_163, x_171, x_160); +x_173 = lean_box(0); +x_174 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__18; +lean_inc(x_24); +x_175 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_175, 0, x_24); lean_ctor_set(x_175, 1, x_174); -x_176 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__29; -x_177 = l_Lean_addMacroScope(x_159, x_176, x_156); -x_178 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__28; -x_179 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__33; -lean_inc(x_20); -x_180 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_180, 0, x_20); -lean_ctor_set(x_180, 1, x_178); -lean_ctor_set(x_180, 2, x_177); -lean_ctor_set(x_180, 3, x_179); -lean_inc(x_20); -x_181 = l_Lean_Syntax_node1(x_20, x_162, x_2); -x_182 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__26; -lean_inc(x_20); -x_183 = l_Lean_Syntax_node2(x_20, x_182, x_180, x_181); -x_184 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__23; -lean_inc(x_20); -x_185 = l_Lean_Syntax_node2(x_20, x_184, x_175, x_183); -lean_inc(x_20); -x_186 = l_Lean_Syntax_node1(x_20, x_162, x_185); -x_187 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__21; -lean_inc(x_164); -lean_inc(x_20); -x_188 = l_Lean_Syntax_node2(x_20, x_187, x_164, x_186); -x_189 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1; -lean_inc(x_20); +lean_ctor_set(x_175, 2, x_172); +lean_ctor_set(x_175, 3, x_173); +x_176 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__16; +lean_inc(x_168); +lean_inc(x_24); +x_177 = l_Lean_Syntax_node2(x_24, x_176, x_175, x_168); +x_178 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__24; +lean_inc(x_24); +x_179 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_179, 0, x_24); +lean_ctor_set(x_179, 1, x_178); +x_180 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__29; +x_181 = l_Lean_addMacroScope(x_163, x_180, x_160); +x_182 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__28; +x_183 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__33; +lean_inc(x_24); +x_184 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_184, 0, x_24); +lean_ctor_set(x_184, 1, x_182); +lean_ctor_set(x_184, 2, x_181); +lean_ctor_set(x_184, 3, x_183); +lean_inc(x_24); +x_185 = l_Lean_Syntax_node1(x_24, x_166, x_2); +x_186 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__26; +lean_inc(x_24); +x_187 = l_Lean_Syntax_node2(x_24, x_186, x_184, x_185); +x_188 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__23; +lean_inc(x_24); +x_189 = l_Lean_Syntax_node2(x_24, x_188, x_179, x_187); +lean_inc(x_24); +x_190 = l_Lean_Syntax_node1(x_24, x_166, x_189); +x_191 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__21; +lean_inc(x_168); +lean_inc(x_24); +x_192 = l_Lean_Syntax_node2(x_24, x_191, x_168, x_190); +x_193 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__43; +lean_inc(x_24); +lean_ctor_set_tag(x_19, 2); +lean_ctor_set(x_19, 1, x_193); +lean_ctor_set(x_19, 0, x_24); +x_194 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__3; +lean_inc(x_24); lean_ctor_set_tag(x_15, 2); -lean_ctor_set(x_15, 1, x_189); -lean_ctor_set(x_15, 0, x_20); -x_190 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__3; -lean_inc(x_20); -lean_ctor_set_tag(x_11, 2); -lean_ctor_set(x_11, 1, x_190); -lean_ctor_set(x_11, 0, x_20); -x_191 = lean_mk_syntax_ident(x_6); -x_192 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__43; -lean_inc(x_20); -x_193 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_193, 0, x_20); -lean_ctor_set(x_193, 1, x_192); -x_194 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__44; -lean_inc(x_20); -x_195 = l_Lean_Syntax_node2(x_20, x_194, x_193, x_3); -x_196 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__2; -lean_inc(x_164); -lean_inc(x_20); -x_197 = l_Lean_Syntax_node4(x_20, x_196, x_11, x_164, x_191, x_195); -x_198 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__47; -lean_inc_n(x_164, 2); -lean_inc(x_20); -x_199 = l_Lean_Syntax_node2(x_20, x_198, x_164, x_164); -x_200 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__42; -lean_inc(x_164); -lean_inc(x_20); -x_201 = l_Lean_Syntax_node4(x_20, x_200, x_15, x_197, x_199, x_164); -x_202 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__9; -lean_inc(x_164); -lean_inc(x_20); -x_203 = l_Lean_Syntax_node5(x_20, x_202, x_166, x_173, x_188, x_201, x_164); +lean_ctor_set(x_15, 1, x_194); +lean_ctor_set(x_15, 0, x_24); +x_195 = lean_mk_syntax_ident(x_6); +x_196 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__44; +lean_inc(x_24); +x_197 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_197, 0, x_24); +lean_ctor_set(x_197, 1, x_196); +x_198 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__45; +lean_inc(x_24); +x_199 = l_Lean_Syntax_node2(x_24, x_198, x_197, x_3); +x_200 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__2; +lean_inc(x_168); +lean_inc(x_24); +x_201 = l_Lean_Syntax_node4(x_24, x_200, x_15, x_168, x_195, x_199); +x_202 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48; +lean_inc_n(x_168, 2); +lean_inc(x_24); +x_203 = l_Lean_Syntax_node2(x_24, x_202, x_168, x_168); +x_204 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__42; +lean_inc(x_168); +lean_inc(x_24); +x_205 = l_Lean_Syntax_node4(x_24, x_204, x_19, x_201, x_203, x_168); +x_206 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__9; +lean_inc(x_168); +lean_inc(x_24); +x_207 = l_Lean_Syntax_node5(x_24, x_206, x_170, x_177, x_192, x_205, x_168); if (lean_obj_tag(x_4) == 0) { -lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; -x_204 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48; -lean_inc(x_20); -x_205 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_205, 0, x_20); -lean_ctor_set(x_205, 1, x_162); -lean_ctor_set(x_205, 2, x_204); -lean_inc_n(x_164, 4); -lean_inc(x_20); -x_206 = l_Lean_Syntax_node6(x_20, x_5, x_164, x_164, x_164, x_164, x_205, x_164); -x_207 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; -lean_inc(x_20); -x_208 = l_Lean_Syntax_node2(x_20, x_207, x_206, x_203); -x_209 = l_Lean_Syntax_node2(x_20, x_162, x_208, x_1); -x_210 = l_Lean_Elab_Command_elabCommand(x_209, x_8, x_9, x_160); -return x_210; -} -else -{ -lean_object* x_211; uint8_t x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; -x_211 = lean_ctor_get(x_4, 0); -x_212 = 1; -x_213 = l_Lean_SourceInfo_fromRef(x_211, x_212); -x_214 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__4; -x_215 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_215, 0, x_213); -lean_ctor_set(x_215, 1, x_214); -x_216 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__5; -lean_inc(x_20); -x_217 = l_Lean_Syntax_node1(x_20, x_216, x_215); -x_218 = l_Array_mkArray1___rarg(x_217); -x_219 = l_Array_append___rarg(x_163, x_218); -lean_dec(x_218); -lean_inc(x_20); -x_220 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_220, 0, x_20); -lean_ctor_set(x_220, 1, x_162); -lean_ctor_set(x_220, 2, x_219); -lean_inc_n(x_164, 4); -lean_inc(x_20); -x_221 = l_Lean_Syntax_node6(x_20, x_5, x_164, x_164, x_164, x_164, x_220, x_164); -x_222 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; -lean_inc(x_20); -x_223 = l_Lean_Syntax_node2(x_20, x_222, x_221, x_203); -x_224 = l_Lean_Syntax_node2(x_20, x_162, x_223, x_1); -x_225 = l_Lean_Elab_Command_elabCommand(x_224, x_8, x_9, x_160); -return x_225; +lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; +x_208 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__49; +lean_inc(x_24); +x_209 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_209, 0, x_24); +lean_ctor_set(x_209, 1, x_166); +lean_ctor_set(x_209, 2, x_208); +lean_inc_n(x_168, 4); +lean_inc(x_24); +x_210 = l_Lean_Syntax_node6(x_24, x_5, x_168, x_168, x_168, x_168, x_209, x_168); +x_211 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; +lean_inc(x_24); +x_212 = l_Lean_Syntax_node2(x_24, x_211, x_210, x_207); +x_213 = l_Lean_Syntax_node2(x_24, x_166, x_212, x_1); +x_214 = l_Lean_Elab_Command_elabCommand(x_213, x_8, x_9, x_164); +return x_214; +} +else +{ +lean_object* x_215; uint8_t x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; +x_215 = lean_ctor_get(x_4, 0); +x_216 = 1; +x_217 = l_Lean_SourceInfo_fromRef(x_215, x_216); +x_218 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__4; +x_219 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_219, 0, x_217); +lean_ctor_set(x_219, 1, x_218); +x_220 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__5; +lean_inc(x_24); +x_221 = l_Lean_Syntax_node1(x_24, x_220, x_219); +x_222 = l_Array_mkArray1___rarg(x_221); +x_223 = l_Array_append___rarg(x_167, x_222); +lean_dec(x_222); +lean_inc(x_24); +x_224 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_224, 0, x_24); +lean_ctor_set(x_224, 1, x_166); +lean_ctor_set(x_224, 2, x_223); +lean_inc_n(x_168, 4); +lean_inc(x_24); +x_225 = l_Lean_Syntax_node6(x_24, x_5, x_168, x_168, x_168, x_168, x_224, x_168); +x_226 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; +lean_inc(x_24); +x_227 = l_Lean_Syntax_node2(x_24, x_226, x_225, x_207); +x_228 = l_Lean_Syntax_node2(x_24, x_166, x_227, x_1); +x_229 = l_Lean_Elab_Command_elabCommand(x_228, x_8, x_9, x_164); +return x_229; } } } else { -lean_object* x_226; lean_object* x_227; uint8_t x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; -x_226 = lean_ctor_get(x_15, 0); -x_227 = lean_ctor_get(x_15, 1); -lean_inc(x_227); -lean_inc(x_226); -lean_dec(x_15); -x_228 = 0; -x_229 = l_Lean_SourceInfo_fromRef(x_226, x_228); -lean_dec(x_226); -x_230 = l_Lean_Elab_Command_getCurrMacroScope(x_8, x_9, x_227); -x_231 = lean_ctor_get(x_230, 0); +lean_object* x_230; lean_object* x_231; uint8_t x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; +x_230 = lean_ctor_get(x_19, 0); +x_231 = lean_ctor_get(x_19, 1); lean_inc(x_231); -x_232 = lean_ctor_get(x_230, 1); -lean_inc(x_232); -if (lean_is_exclusive(x_230)) { - lean_ctor_release(x_230, 0); - lean_ctor_release(x_230, 1); - x_233 = x_230; -} else { - lean_dec_ref(x_230); - x_233 = lean_box(0); -} -x_234 = l_Lean_Elab_Command_getMainModule___rarg(x_9, x_232); +lean_inc(x_230); +lean_dec(x_19); +x_232 = 0; +x_233 = l_Lean_SourceInfo_fromRef(x_230, x_232); +lean_dec(x_230); +x_234 = l_Lean_Elab_Command_getCurrMacroScope(x_8, x_9, x_231); x_235 = lean_ctor_get(x_234, 0); lean_inc(x_235); x_236 = lean_ctor_get(x_234, 1); @@ -12899,196 +10672,196 @@ if (lean_is_exclusive(x_234)) { lean_dec_ref(x_234); x_237 = lean_box(0); } -x_238 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; -x_239 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; -lean_inc(x_229); -x_240 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_240, 0, x_229); -lean_ctor_set(x_240, 1, x_238); -lean_ctor_set(x_240, 2, x_239); -x_241 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__14; -lean_inc(x_229); -if (lean_is_scalar(x_237)) { - x_242 = lean_alloc_ctor(2, 2, 0); -} else { - x_242 = x_237; - lean_ctor_set_tag(x_242, 2); -} -lean_ctor_set(x_242, 0, x_229); -lean_ctor_set(x_242, 1, x_241); -x_243 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__19; -lean_inc(x_231); -lean_inc(x_235); -x_244 = l_Lean_addMacroScope(x_235, x_243, x_231); -x_245 = lean_box(0); -x_246 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__18; -lean_inc(x_229); -x_247 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_247, 0, x_229); -lean_ctor_set(x_247, 1, x_246); -lean_ctor_set(x_247, 2, x_244); -lean_ctor_set(x_247, 3, x_245); -x_248 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__16; +x_238 = l_Lean_Elab_Command_getMainModule___rarg(x_9, x_236); +x_239 = lean_ctor_get(x_238, 0); +lean_inc(x_239); +x_240 = lean_ctor_get(x_238, 1); lean_inc(x_240); -lean_inc(x_229); -x_249 = l_Lean_Syntax_node2(x_229, x_248, x_247, x_240); -x_250 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__24; -lean_inc(x_229); -if (lean_is_scalar(x_233)) { - x_251 = lean_alloc_ctor(2, 2, 0); +if (lean_is_exclusive(x_238)) { + lean_ctor_release(x_238, 0); + lean_ctor_release(x_238, 1); + x_241 = x_238; } else { - x_251 = x_233; - lean_ctor_set_tag(x_251, 2); + lean_dec_ref(x_238); + x_241 = lean_box(0); +} +x_242 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; +x_243 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; +lean_inc(x_233); +x_244 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_244, 0, x_233); +lean_ctor_set(x_244, 1, x_242); +lean_ctor_set(x_244, 2, x_243); +x_245 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__14; +lean_inc(x_233); +if (lean_is_scalar(x_241)) { + x_246 = lean_alloc_ctor(2, 2, 0); +} else { + x_246 = x_241; + lean_ctor_set_tag(x_246, 2); } -lean_ctor_set(x_251, 0, x_229); +lean_ctor_set(x_246, 0, x_233); +lean_ctor_set(x_246, 1, x_245); +x_247 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__19; +lean_inc(x_235); +lean_inc(x_239); +x_248 = l_Lean_addMacroScope(x_239, x_247, x_235); +x_249 = lean_box(0); +x_250 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__18; +lean_inc(x_233); +x_251 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_251, 0, x_233); lean_ctor_set(x_251, 1, x_250); -x_252 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__29; -x_253 = l_Lean_addMacroScope(x_235, x_252, x_231); -x_254 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__28; -x_255 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__33; -lean_inc(x_229); -x_256 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_256, 0, x_229); -lean_ctor_set(x_256, 1, x_254); -lean_ctor_set(x_256, 2, x_253); -lean_ctor_set(x_256, 3, x_255); -lean_inc(x_229); -x_257 = l_Lean_Syntax_node1(x_229, x_238, x_2); -x_258 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__26; -lean_inc(x_229); -x_259 = l_Lean_Syntax_node2(x_229, x_258, x_256, x_257); -x_260 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__23; -lean_inc(x_229); -x_261 = l_Lean_Syntax_node2(x_229, x_260, x_251, x_259); -lean_inc(x_229); -x_262 = l_Lean_Syntax_node1(x_229, x_238, x_261); -x_263 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__21; -lean_inc(x_240); -lean_inc(x_229); -x_264 = l_Lean_Syntax_node2(x_229, x_263, x_240, x_262); -x_265 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1; -lean_inc(x_229); -x_266 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_266, 0, x_229); -lean_ctor_set(x_266, 1, x_265); -x_267 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__3; -lean_inc(x_229); -lean_ctor_set_tag(x_11, 2); -lean_ctor_set(x_11, 1, x_267); -lean_ctor_set(x_11, 0, x_229); -x_268 = lean_mk_syntax_ident(x_6); +lean_ctor_set(x_251, 2, x_248); +lean_ctor_set(x_251, 3, x_249); +x_252 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__16; +lean_inc(x_244); +lean_inc(x_233); +x_253 = l_Lean_Syntax_node2(x_233, x_252, x_251, x_244); +x_254 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__24; +lean_inc(x_233); +if (lean_is_scalar(x_237)) { + x_255 = lean_alloc_ctor(2, 2, 0); +} else { + x_255 = x_237; + lean_ctor_set_tag(x_255, 2); +} +lean_ctor_set(x_255, 0, x_233); +lean_ctor_set(x_255, 1, x_254); +x_256 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__29; +x_257 = l_Lean_addMacroScope(x_239, x_256, x_235); +x_258 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__28; +x_259 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__33; +lean_inc(x_233); +x_260 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_260, 0, x_233); +lean_ctor_set(x_260, 1, x_258); +lean_ctor_set(x_260, 2, x_257); +lean_ctor_set(x_260, 3, x_259); +lean_inc(x_233); +x_261 = l_Lean_Syntax_node1(x_233, x_242, x_2); +x_262 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__26; +lean_inc(x_233); +x_263 = l_Lean_Syntax_node2(x_233, x_262, x_260, x_261); +x_264 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__23; +lean_inc(x_233); +x_265 = l_Lean_Syntax_node2(x_233, x_264, x_255, x_263); +lean_inc(x_233); +x_266 = l_Lean_Syntax_node1(x_233, x_242, x_265); +x_267 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__21; +lean_inc(x_244); +lean_inc(x_233); +x_268 = l_Lean_Syntax_node2(x_233, x_267, x_244, x_266); x_269 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__43; -lean_inc(x_229); +lean_inc(x_233); x_270 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_270, 0, x_229); +lean_ctor_set(x_270, 0, x_233); lean_ctor_set(x_270, 1, x_269); -x_271 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__44; -lean_inc(x_229); -x_272 = l_Lean_Syntax_node2(x_229, x_271, x_270, x_3); -x_273 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__2; -lean_inc(x_240); -lean_inc(x_229); -x_274 = l_Lean_Syntax_node4(x_229, x_273, x_11, x_240, x_268, x_272); -x_275 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__47; -lean_inc_n(x_240, 2); -lean_inc(x_229); -x_276 = l_Lean_Syntax_node2(x_229, x_275, x_240, x_240); -x_277 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__42; -lean_inc(x_240); -lean_inc(x_229); -x_278 = l_Lean_Syntax_node4(x_229, x_277, x_266, x_274, x_276, x_240); -x_279 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__9; -lean_inc(x_240); -lean_inc(x_229); -x_280 = l_Lean_Syntax_node5(x_229, x_279, x_242, x_249, x_264, x_278, x_240); +x_271 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__3; +lean_inc(x_233); +lean_ctor_set_tag(x_15, 2); +lean_ctor_set(x_15, 1, x_271); +lean_ctor_set(x_15, 0, x_233); +x_272 = lean_mk_syntax_ident(x_6); +x_273 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__44; +lean_inc(x_233); +x_274 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_274, 0, x_233); +lean_ctor_set(x_274, 1, x_273); +x_275 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__45; +lean_inc(x_233); +x_276 = l_Lean_Syntax_node2(x_233, x_275, x_274, x_3); +x_277 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__2; +lean_inc(x_244); +lean_inc(x_233); +x_278 = l_Lean_Syntax_node4(x_233, x_277, x_15, x_244, x_272, x_276); +x_279 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48; +lean_inc_n(x_244, 2); +lean_inc(x_233); +x_280 = l_Lean_Syntax_node2(x_233, x_279, x_244, x_244); +x_281 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__42; +lean_inc(x_244); +lean_inc(x_233); +x_282 = l_Lean_Syntax_node4(x_233, x_281, x_270, x_278, x_280, x_244); +x_283 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__9; +lean_inc(x_244); +lean_inc(x_233); +x_284 = l_Lean_Syntax_node5(x_233, x_283, x_246, x_253, x_268, x_282, x_244); if (lean_obj_tag(x_4) == 0) { -lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; lean_object* x_286; lean_object* x_287; -x_281 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48; -lean_inc(x_229); -x_282 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_282, 0, x_229); -lean_ctor_set(x_282, 1, x_238); -lean_ctor_set(x_282, 2, x_281); -lean_inc_n(x_240, 4); -lean_inc(x_229); -x_283 = l_Lean_Syntax_node6(x_229, x_5, x_240, x_240, x_240, x_240, x_282, x_240); -x_284 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; -lean_inc(x_229); -x_285 = l_Lean_Syntax_node2(x_229, x_284, x_283, x_280); -x_286 = l_Lean_Syntax_node2(x_229, x_238, x_285, x_1); -x_287 = l_Lean_Elab_Command_elabCommand(x_286, x_8, x_9, x_236); -return x_287; -} -else -{ -lean_object* x_288; uint8_t x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; lean_object* x_294; lean_object* x_295; lean_object* x_296; lean_object* x_297; lean_object* x_298; lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; -x_288 = lean_ctor_get(x_4, 0); -x_289 = 1; -x_290 = l_Lean_SourceInfo_fromRef(x_288, x_289); -x_291 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__4; -x_292 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_292, 0, x_290); -lean_ctor_set(x_292, 1, x_291); -x_293 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__5; -lean_inc(x_229); -x_294 = l_Lean_Syntax_node1(x_229, x_293, x_292); -x_295 = l_Array_mkArray1___rarg(x_294); -x_296 = l_Array_append___rarg(x_239, x_295); -lean_dec(x_295); -lean_inc(x_229); -x_297 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_297, 0, x_229); -lean_ctor_set(x_297, 1, x_238); -lean_ctor_set(x_297, 2, x_296); -lean_inc_n(x_240, 4); -lean_inc(x_229); -x_298 = l_Lean_Syntax_node6(x_229, x_5, x_240, x_240, x_240, x_240, x_297, x_240); -x_299 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; -lean_inc(x_229); -x_300 = l_Lean_Syntax_node2(x_229, x_299, x_298, x_280); -x_301 = l_Lean_Syntax_node2(x_229, x_238, x_300, x_1); -x_302 = l_Lean_Elab_Command_elabCommand(x_301, x_8, x_9, x_236); -return x_302; -} -} -} -else -{ -lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; lean_object* x_307; uint8_t x_308; lean_object* x_309; lean_object* x_310; lean_object* x_311; lean_object* x_312; lean_object* x_313; lean_object* x_314; lean_object* x_315; lean_object* x_316; lean_object* x_317; lean_object* x_318; lean_object* x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; lean_object* x_324; lean_object* x_325; lean_object* x_326; lean_object* x_327; lean_object* x_328; lean_object* x_329; lean_object* x_330; lean_object* x_331; lean_object* x_332; lean_object* x_333; lean_object* x_334; lean_object* x_335; lean_object* x_336; lean_object* x_337; lean_object* x_338; lean_object* x_339; lean_object* x_340; lean_object* x_341; lean_object* x_342; lean_object* x_343; lean_object* x_344; lean_object* x_345; lean_object* x_346; lean_object* x_347; lean_object* x_348; lean_object* x_349; lean_object* x_350; lean_object* x_351; lean_object* x_352; lean_object* x_353; lean_object* x_354; lean_object* x_355; lean_object* x_356; lean_object* x_357; lean_object* x_358; lean_object* x_359; lean_object* x_360; lean_object* x_361; -x_303 = lean_ctor_get(x_11, 1); -lean_inc(x_303); -lean_dec(x_11); -x_304 = l_Lean_Elab_Command_getRef(x_8, x_9, x_303); -x_305 = lean_ctor_get(x_304, 0); -lean_inc(x_305); -x_306 = lean_ctor_get(x_304, 1); -lean_inc(x_306); -if (lean_is_exclusive(x_304)) { - lean_ctor_release(x_304, 0); - lean_ctor_release(x_304, 1); - x_307 = x_304; -} else { - lean_dec_ref(x_304); - x_307 = lean_box(0); -} -x_308 = 0; -x_309 = l_Lean_SourceInfo_fromRef(x_305, x_308); -lean_dec(x_305); -x_310 = l_Lean_Elab_Command_getCurrMacroScope(x_8, x_9, x_306); -x_311 = lean_ctor_get(x_310, 0); -lean_inc(x_311); -x_312 = lean_ctor_get(x_310, 1); -lean_inc(x_312); -if (lean_is_exclusive(x_310)) { - lean_ctor_release(x_310, 0); - lean_ctor_release(x_310, 1); - x_313 = x_310; +lean_object* x_285; lean_object* x_286; lean_object* x_287; lean_object* x_288; lean_object* x_289; lean_object* x_290; lean_object* x_291; +x_285 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__49; +lean_inc(x_233); +x_286 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_286, 0, x_233); +lean_ctor_set(x_286, 1, x_242); +lean_ctor_set(x_286, 2, x_285); +lean_inc_n(x_244, 4); +lean_inc(x_233); +x_287 = l_Lean_Syntax_node6(x_233, x_5, x_244, x_244, x_244, x_244, x_286, x_244); +x_288 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; +lean_inc(x_233); +x_289 = l_Lean_Syntax_node2(x_233, x_288, x_287, x_284); +x_290 = l_Lean_Syntax_node2(x_233, x_242, x_289, x_1); +x_291 = l_Lean_Elab_Command_elabCommand(x_290, x_8, x_9, x_240); +return x_291; +} +else +{ +lean_object* x_292; uint8_t x_293; lean_object* x_294; lean_object* x_295; lean_object* x_296; lean_object* x_297; lean_object* x_298; lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; +x_292 = lean_ctor_get(x_4, 0); +x_293 = 1; +x_294 = l_Lean_SourceInfo_fromRef(x_292, x_293); +x_295 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__4; +x_296 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_296, 0, x_294); +lean_ctor_set(x_296, 1, x_295); +x_297 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__5; +lean_inc(x_233); +x_298 = l_Lean_Syntax_node1(x_233, x_297, x_296); +x_299 = l_Array_mkArray1___rarg(x_298); +x_300 = l_Array_append___rarg(x_243, x_299); +lean_dec(x_299); +lean_inc(x_233); +x_301 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_301, 0, x_233); +lean_ctor_set(x_301, 1, x_242); +lean_ctor_set(x_301, 2, x_300); +lean_inc_n(x_244, 4); +lean_inc(x_233); +x_302 = l_Lean_Syntax_node6(x_233, x_5, x_244, x_244, x_244, x_244, x_301, x_244); +x_303 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; +lean_inc(x_233); +x_304 = l_Lean_Syntax_node2(x_233, x_303, x_302, x_284); +x_305 = l_Lean_Syntax_node2(x_233, x_242, x_304, x_1); +x_306 = l_Lean_Elab_Command_elabCommand(x_305, x_8, x_9, x_240); +return x_306; +} +} +} +else +{ +lean_object* x_307; lean_object* x_308; lean_object* x_309; lean_object* x_310; lean_object* x_311; uint8_t x_312; lean_object* x_313; lean_object* x_314; lean_object* x_315; lean_object* x_316; lean_object* x_317; lean_object* x_318; lean_object* x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; lean_object* x_324; lean_object* x_325; lean_object* x_326; lean_object* x_327; lean_object* x_328; lean_object* x_329; lean_object* x_330; lean_object* x_331; lean_object* x_332; lean_object* x_333; lean_object* x_334; lean_object* x_335; lean_object* x_336; lean_object* x_337; lean_object* x_338; lean_object* x_339; lean_object* x_340; lean_object* x_341; lean_object* x_342; lean_object* x_343; lean_object* x_344; lean_object* x_345; lean_object* x_346; lean_object* x_347; lean_object* x_348; lean_object* x_349; lean_object* x_350; lean_object* x_351; lean_object* x_352; lean_object* x_353; lean_object* x_354; lean_object* x_355; lean_object* x_356; lean_object* x_357; lean_object* x_358; lean_object* x_359; lean_object* x_360; lean_object* x_361; lean_object* x_362; lean_object* x_363; lean_object* x_364; lean_object* x_365; +x_307 = lean_ctor_get(x_15, 1); +lean_inc(x_307); +lean_dec(x_15); +x_308 = l_Lean_Elab_Command_getRef(x_8, x_9, x_307); +x_309 = lean_ctor_get(x_308, 0); +lean_inc(x_309); +x_310 = lean_ctor_get(x_308, 1); +lean_inc(x_310); +if (lean_is_exclusive(x_308)) { + lean_ctor_release(x_308, 0); + lean_ctor_release(x_308, 1); + x_311 = x_308; } else { - lean_dec_ref(x_310); - x_313 = lean_box(0); + lean_dec_ref(x_308); + x_311 = lean_box(0); } -x_314 = l_Lean_Elab_Command_getMainModule___rarg(x_9, x_312); +x_312 = 0; +x_313 = l_Lean_SourceInfo_fromRef(x_309, x_312); +lean_dec(x_309); +x_314 = l_Lean_Elab_Command_getCurrMacroScope(x_8, x_9, x_310); x_315 = lean_ctor_get(x_314, 0); lean_inc(x_315); x_316 = lean_ctor_get(x_314, 1); @@ -13101,162 +10874,175 @@ if (lean_is_exclusive(x_314)) { lean_dec_ref(x_314); x_317 = lean_box(0); } -x_318 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; -x_319 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; -lean_inc(x_309); -x_320 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_320, 0, x_309); -lean_ctor_set(x_320, 1, x_318); -lean_ctor_set(x_320, 2, x_319); -x_321 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__14; -lean_inc(x_309); -if (lean_is_scalar(x_317)) { - x_322 = lean_alloc_ctor(2, 2, 0); -} else { - x_322 = x_317; - lean_ctor_set_tag(x_322, 2); -} -lean_ctor_set(x_322, 0, x_309); -lean_ctor_set(x_322, 1, x_321); -x_323 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__19; -lean_inc(x_311); -lean_inc(x_315); -x_324 = l_Lean_addMacroScope(x_315, x_323, x_311); -x_325 = lean_box(0); -x_326 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__18; -lean_inc(x_309); -x_327 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_327, 0, x_309); -lean_ctor_set(x_327, 1, x_326); -lean_ctor_set(x_327, 2, x_324); -lean_ctor_set(x_327, 3, x_325); -x_328 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__16; +x_318 = l_Lean_Elab_Command_getMainModule___rarg(x_9, x_316); +x_319 = lean_ctor_get(x_318, 0); +lean_inc(x_319); +x_320 = lean_ctor_get(x_318, 1); lean_inc(x_320); -lean_inc(x_309); -x_329 = l_Lean_Syntax_node2(x_309, x_328, x_327, x_320); -x_330 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__24; -lean_inc(x_309); -if (lean_is_scalar(x_313)) { - x_331 = lean_alloc_ctor(2, 2, 0); +if (lean_is_exclusive(x_318)) { + lean_ctor_release(x_318, 0); + lean_ctor_release(x_318, 1); + x_321 = x_318; +} else { + lean_dec_ref(x_318); + x_321 = lean_box(0); +} +x_322 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; +x_323 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; +lean_inc(x_313); +x_324 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_324, 0, x_313); +lean_ctor_set(x_324, 1, x_322); +lean_ctor_set(x_324, 2, x_323); +x_325 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__14; +lean_inc(x_313); +if (lean_is_scalar(x_321)) { + x_326 = lean_alloc_ctor(2, 2, 0); } else { - x_331 = x_313; - lean_ctor_set_tag(x_331, 2); + x_326 = x_321; + lean_ctor_set_tag(x_326, 2); } -lean_ctor_set(x_331, 0, x_309); +lean_ctor_set(x_326, 0, x_313); +lean_ctor_set(x_326, 1, x_325); +x_327 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__19; +lean_inc(x_315); +lean_inc(x_319); +x_328 = l_Lean_addMacroScope(x_319, x_327, x_315); +x_329 = lean_box(0); +x_330 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__18; +lean_inc(x_313); +x_331 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_331, 0, x_313); lean_ctor_set(x_331, 1, x_330); -x_332 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__29; -x_333 = l_Lean_addMacroScope(x_315, x_332, x_311); -x_334 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__28; -x_335 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__33; -lean_inc(x_309); -x_336 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_336, 0, x_309); -lean_ctor_set(x_336, 1, x_334); -lean_ctor_set(x_336, 2, x_333); -lean_ctor_set(x_336, 3, x_335); -lean_inc(x_309); -x_337 = l_Lean_Syntax_node1(x_309, x_318, x_2); -x_338 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__26; -lean_inc(x_309); -x_339 = l_Lean_Syntax_node2(x_309, x_338, x_336, x_337); -x_340 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__23; -lean_inc(x_309); -x_341 = l_Lean_Syntax_node2(x_309, x_340, x_331, x_339); -lean_inc(x_309); -x_342 = l_Lean_Syntax_node1(x_309, x_318, x_341); -x_343 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__21; -lean_inc(x_320); -lean_inc(x_309); -x_344 = l_Lean_Syntax_node2(x_309, x_343, x_320, x_342); -x_345 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1; -lean_inc(x_309); -if (lean_is_scalar(x_307)) { - x_346 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_331, 2, x_328); +lean_ctor_set(x_331, 3, x_329); +x_332 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__16; +lean_inc(x_324); +lean_inc(x_313); +x_333 = l_Lean_Syntax_node2(x_313, x_332, x_331, x_324); +x_334 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__24; +lean_inc(x_313); +if (lean_is_scalar(x_317)) { + x_335 = lean_alloc_ctor(2, 2, 0); } else { - x_346 = x_307; - lean_ctor_set_tag(x_346, 2); -} -lean_ctor_set(x_346, 0, x_309); -lean_ctor_set(x_346, 1, x_345); -x_347 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__3; -lean_inc(x_309); -x_348 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_348, 0, x_309); -lean_ctor_set(x_348, 1, x_347); -x_349 = lean_mk_syntax_ident(x_6); -x_350 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__43; -lean_inc(x_309); -x_351 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_351, 0, x_309); -lean_ctor_set(x_351, 1, x_350); -x_352 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__44; -lean_inc(x_309); -x_353 = l_Lean_Syntax_node2(x_309, x_352, x_351, x_3); -x_354 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__2; -lean_inc(x_320); -lean_inc(x_309); -x_355 = l_Lean_Syntax_node4(x_309, x_354, x_348, x_320, x_349, x_353); -x_356 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__47; -lean_inc_n(x_320, 2); -lean_inc(x_309); -x_357 = l_Lean_Syntax_node2(x_309, x_356, x_320, x_320); -x_358 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__42; -lean_inc(x_320); -lean_inc(x_309); -x_359 = l_Lean_Syntax_node4(x_309, x_358, x_346, x_355, x_357, x_320); -x_360 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__9; -lean_inc(x_320); -lean_inc(x_309); -x_361 = l_Lean_Syntax_node5(x_309, x_360, x_322, x_329, x_344, x_359, x_320); + x_335 = x_317; + lean_ctor_set_tag(x_335, 2); +} +lean_ctor_set(x_335, 0, x_313); +lean_ctor_set(x_335, 1, x_334); +x_336 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__29; +x_337 = l_Lean_addMacroScope(x_319, x_336, x_315); +x_338 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__28; +x_339 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__33; +lean_inc(x_313); +x_340 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_340, 0, x_313); +lean_ctor_set(x_340, 1, x_338); +lean_ctor_set(x_340, 2, x_337); +lean_ctor_set(x_340, 3, x_339); +lean_inc(x_313); +x_341 = l_Lean_Syntax_node1(x_313, x_322, x_2); +x_342 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__26; +lean_inc(x_313); +x_343 = l_Lean_Syntax_node2(x_313, x_342, x_340, x_341); +x_344 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__23; +lean_inc(x_313); +x_345 = l_Lean_Syntax_node2(x_313, x_344, x_335, x_343); +lean_inc(x_313); +x_346 = l_Lean_Syntax_node1(x_313, x_322, x_345); +x_347 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__21; +lean_inc(x_324); +lean_inc(x_313); +x_348 = l_Lean_Syntax_node2(x_313, x_347, x_324, x_346); +x_349 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__43; +lean_inc(x_313); +if (lean_is_scalar(x_311)) { + x_350 = lean_alloc_ctor(2, 2, 0); +} else { + x_350 = x_311; + lean_ctor_set_tag(x_350, 2); +} +lean_ctor_set(x_350, 0, x_313); +lean_ctor_set(x_350, 1, x_349); +x_351 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__3; +lean_inc(x_313); +x_352 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_352, 0, x_313); +lean_ctor_set(x_352, 1, x_351); +x_353 = lean_mk_syntax_ident(x_6); +x_354 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__44; +lean_inc(x_313); +x_355 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_355, 0, x_313); +lean_ctor_set(x_355, 1, x_354); +x_356 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__45; +lean_inc(x_313); +x_357 = l_Lean_Syntax_node2(x_313, x_356, x_355, x_3); +x_358 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__2; +lean_inc(x_324); +lean_inc(x_313); +x_359 = l_Lean_Syntax_node4(x_313, x_358, x_352, x_324, x_353, x_357); +x_360 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48; +lean_inc_n(x_324, 2); +lean_inc(x_313); +x_361 = l_Lean_Syntax_node2(x_313, x_360, x_324, x_324); +x_362 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__42; +lean_inc(x_324); +lean_inc(x_313); +x_363 = l_Lean_Syntax_node4(x_313, x_362, x_350, x_359, x_361, x_324); +x_364 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__9; +lean_inc(x_324); +lean_inc(x_313); +x_365 = l_Lean_Syntax_node5(x_313, x_364, x_326, x_333, x_348, x_363, x_324); if (lean_obj_tag(x_4) == 0) { -lean_object* x_362; lean_object* x_363; lean_object* x_364; lean_object* x_365; lean_object* x_366; lean_object* x_367; lean_object* x_368; -x_362 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48; -lean_inc(x_309); -x_363 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_363, 0, x_309); -lean_ctor_set(x_363, 1, x_318); -lean_ctor_set(x_363, 2, x_362); -lean_inc_n(x_320, 4); -lean_inc(x_309); -x_364 = l_Lean_Syntax_node6(x_309, x_5, x_320, x_320, x_320, x_320, x_363, x_320); -x_365 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; -lean_inc(x_309); -x_366 = l_Lean_Syntax_node2(x_309, x_365, x_364, x_361); -x_367 = l_Lean_Syntax_node2(x_309, x_318, x_366, x_1); -x_368 = l_Lean_Elab_Command_elabCommand(x_367, x_8, x_9, x_316); -return x_368; -} -else -{ -lean_object* x_369; uint8_t x_370; lean_object* x_371; lean_object* x_372; lean_object* x_373; lean_object* x_374; lean_object* x_375; lean_object* x_376; lean_object* x_377; lean_object* x_378; lean_object* x_379; lean_object* x_380; lean_object* x_381; lean_object* x_382; lean_object* x_383; -x_369 = lean_ctor_get(x_4, 0); -x_370 = 1; -x_371 = l_Lean_SourceInfo_fromRef(x_369, x_370); -x_372 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__4; -x_373 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_373, 0, x_371); -lean_ctor_set(x_373, 1, x_372); -x_374 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__5; -lean_inc(x_309); -x_375 = l_Lean_Syntax_node1(x_309, x_374, x_373); -x_376 = l_Array_mkArray1___rarg(x_375); -x_377 = l_Array_append___rarg(x_319, x_376); -lean_dec(x_376); -lean_inc(x_309); -x_378 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_378, 0, x_309); -lean_ctor_set(x_378, 1, x_318); -lean_ctor_set(x_378, 2, x_377); -lean_inc_n(x_320, 4); -lean_inc(x_309); -x_379 = l_Lean_Syntax_node6(x_309, x_5, x_320, x_320, x_320, x_320, x_378, x_320); -x_380 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; -lean_inc(x_309); -x_381 = l_Lean_Syntax_node2(x_309, x_380, x_379, x_361); -x_382 = l_Lean_Syntax_node2(x_309, x_318, x_381, x_1); -x_383 = l_Lean_Elab_Command_elabCommand(x_382, x_8, x_9, x_316); -return x_383; +lean_object* x_366; lean_object* x_367; lean_object* x_368; lean_object* x_369; lean_object* x_370; lean_object* x_371; lean_object* x_372; +x_366 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__49; +lean_inc(x_313); +x_367 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_367, 0, x_313); +lean_ctor_set(x_367, 1, x_322); +lean_ctor_set(x_367, 2, x_366); +lean_inc_n(x_324, 4); +lean_inc(x_313); +x_368 = l_Lean_Syntax_node6(x_313, x_5, x_324, x_324, x_324, x_324, x_367, x_324); +x_369 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; +lean_inc(x_313); +x_370 = l_Lean_Syntax_node2(x_313, x_369, x_368, x_365); +x_371 = l_Lean_Syntax_node2(x_313, x_322, x_370, x_1); +x_372 = l_Lean_Elab_Command_elabCommand(x_371, x_8, x_9, x_320); +return x_372; +} +else +{ +lean_object* x_373; uint8_t x_374; lean_object* x_375; lean_object* x_376; lean_object* x_377; lean_object* x_378; lean_object* x_379; lean_object* x_380; lean_object* x_381; lean_object* x_382; lean_object* x_383; lean_object* x_384; lean_object* x_385; lean_object* x_386; lean_object* x_387; +x_373 = lean_ctor_get(x_4, 0); +x_374 = 1; +x_375 = l_Lean_SourceInfo_fromRef(x_373, x_374); +x_376 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__4; +x_377 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_377, 0, x_375); +lean_ctor_set(x_377, 1, x_376); +x_378 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__5; +lean_inc(x_313); +x_379 = l_Lean_Syntax_node1(x_313, x_378, x_377); +x_380 = l_Array_mkArray1___rarg(x_379); +x_381 = l_Array_append___rarg(x_323, x_380); +lean_dec(x_380); +lean_inc(x_313); +x_382 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_382, 0, x_313); +lean_ctor_set(x_382, 1, x_322); +lean_ctor_set(x_382, 2, x_381); +lean_inc_n(x_324, 4); +lean_inc(x_313); +x_383 = l_Lean_Syntax_node6(x_313, x_5, x_324, x_324, x_324, x_324, x_382, x_324); +x_384 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; +lean_inc(x_313); +x_385 = l_Lean_Syntax_node2(x_313, x_384, x_383, x_365); +x_386 = l_Lean_Syntax_node2(x_313, x_322, x_385, x_1); +x_387 = l_Lean_Elab_Command_elabCommand(x_386, x_8, x_9, x_320); +return x_387; } } } @@ -13554,7 +11340,7 @@ x_96 = l_Lean_Syntax_node1(x_44, x_54, x_95); if (lean_obj_tag(x_15) == 0) { lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; -x_97 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48; +x_97 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__49; lean_inc(x_44); x_98 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_98, 0, x_44); @@ -13740,7 +11526,7 @@ x_160 = l_Lean_Syntax_node1(x_44, x_118, x_159); if (lean_obj_tag(x_15) == 0) { lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; -x_161 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48; +x_161 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__49; lean_inc(x_44); x_162 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_162, 0, x_44); @@ -13945,7 +11731,7 @@ x_229 = l_Lean_Syntax_node1(x_44, x_186, x_228); if (lean_obj_tag(x_15) == 0) { lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; -x_230 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48; +x_230 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__49; lean_inc(x_44); x_231 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_231, 0, x_44); @@ -14171,7 +11957,7 @@ x_305 = l_Lean_Syntax_node1(x_250, x_261, x_304); if (lean_obj_tag(x_15) == 0) { lean_object* x_306; lean_object* x_307; lean_object* x_308; lean_object* x_309; lean_object* x_310; -x_306 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48; +x_306 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__49; lean_inc(x_250); x_307 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_307, 0, x_250); @@ -15101,6 +12887,56 @@ return x_36; } } } +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Command_elabInitialize___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Command_elabInitialize___spec__3(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_addDeclarationRanges___at_Lean_Elab_Command_elabInitialize___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; +x_6 = l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabInitialize___spec__4(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___at_Lean_Elab_Command_elabInitialize___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; +x_7 = l_Lean_Elab_addDeclarationRangesFromSyntax___at_Lean_Elab_Command_elabInitialize___spec__2(x_1, x_2, x_3, x_4, x_5, x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Command_elabInitialize___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_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Command_elabInitialize___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_6); +lean_dec(x_4); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Command_elabInitialize___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_addDeclarationRangesForBuiltin___at_Lean_Elab_Command_elabInitialize___spec__1(x_1, x_2, x_3, x_4, x_5, x_6); +lean_dec(x_5); +return x_7; +} +} LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, 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: { @@ -15205,7 +13041,7 @@ x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); return x_6; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__1() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -15215,37 +13051,37 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__2() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__1; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__1; x_2 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__3() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__2; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__2; x_2 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__3; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__4() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__3; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__3; x_2 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__17; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__5() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__5() { _start: { lean_object* x_1; @@ -15253,37 +13089,37 @@ x_1 = lean_mk_string_unchecked("_@", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__6() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__4; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__4; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__5; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__7() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__6; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__6; x_2 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__8() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__7; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__7; x_2 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__9() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__9() { _start: { lean_object* x_1; @@ -15291,17 +13127,17 @@ x_1 = lean_mk_string_unchecked("Declaration", 11, 11); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__10() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__8; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__9; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__8; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__9; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__11() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__11() { _start: { lean_object* x_1; @@ -15309,33 +13145,33 @@ x_1 = lean_mk_string_unchecked("_hyg", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__12() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__10; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__11; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__10; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__11; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__13() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__12; -x_2 = lean_unsigned_to_nat(9024u); +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__12; +x_2 = lean_unsigned_to_nat(7310u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310_(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; x_2 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__7; x_3 = 0; -x_4 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__13; +x_4 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__13; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); return x_5; } @@ -15451,12 +13287,6 @@ l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_setDefName___closed__3 = lean_mark_persistent(l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_setDefName___closed__3); l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_setDefName___closed__4 = _init_l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_setDefName___closed__4(); lean_mark_persistent(l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_setDefName___closed__4); -l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__3___closed__1 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__3___closed__1(); -lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__3___closed__1); -l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___closed__1 = _init_l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___closed__1(); -lean_mark_persistent(l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___closed__1); -l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___closed__2 = _init_l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___closed__2(); -lean_mark_persistent(l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___closed__2); l_Lean_Elab_Command_elabAxiom___lambda__3___closed__1 = _init_l_Lean_Elab_Command_elabAxiom___lambda__3___closed__1(); lean_mark_persistent(l_Lean_Elab_Command_elabAxiom___lambda__3___closed__1); l_Lean_Elab_Command_elabAxiom___lambda__4___closed__1 = _init_l_Lean_Elab_Command_elabAxiom___lambda__4___closed__1(); @@ -15481,64 +13311,6 @@ l_Lean_Elab_Command_elabAxiom___lambda__4___closed__10 = _init_l_Lean_Elab_Comma lean_mark_persistent(l_Lean_Elab_Command_elabAxiom___lambda__4___closed__10); l_Lean_Elab_Command_elabAxiom___lambda__4___closed__11 = _init_l_Lean_Elab_Command_elabAxiom___lambda__4___closed__11(); lean_mark_persistent(l_Lean_Elab_Command_elabAxiom___lambda__4___closed__11); -l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__1___closed__1 = _init_l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__1___closed__1); -l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__1___closed__2 = _init_l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__1___closed__2); -l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__2___closed__1 = _init_l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__2___closed__1(); -lean_mark_persistent(l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__2___closed__1); -l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__2___closed__2 = _init_l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__2___closed__2(); -lean_mark_persistent(l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__2___closed__2); -l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__3___closed__1 = _init_l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__3___closed__1(); -lean_mark_persistent(l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__3___closed__1); -l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__3___closed__2 = _init_l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__3___closed__2(); -lean_mark_persistent(l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__3___closed__2); -l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___closed__1 = _init_l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___closed__1(); -lean_mark_persistent(l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___closed__1); -l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___closed__2 = _init_l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___closed__2(); -lean_mark_persistent(l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___closed__2); -l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__2___closed__1 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__2___closed__1(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__2___closed__1); -l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__2___closed__2 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__2___closed__2(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__2___closed__2); -l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__3___closed__1 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__3___closed__1(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__3___closed__1); -l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__3___closed__2 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__3___closed__2(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__3___closed__2); -l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___closed__1 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___closed__1(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___closed__1); -l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___closed__2 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___closed__2(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___closed__2); -l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___closed__3 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___closed__3(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___closed__3); -l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__1 = _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__1(); -lean_mark_persistent(l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__1); -l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__2 = _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__2(); -lean_mark_persistent(l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__2); -l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__3 = _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__3(); -lean_mark_persistent(l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__3); -l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__4 = _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__4(); -lean_mark_persistent(l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__4); -l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__5 = _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__5(); -lean_mark_persistent(l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__5); -l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__6 = _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__6(); -lean_mark_persistent(l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__6); -l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1 = _init_l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1(); -lean_mark_persistent(l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1); -l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__2 = _init_l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__2(); -lean_mark_persistent(l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__2); -l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__3 = _init_l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__3(); -lean_mark_persistent(l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__3); -l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__4 = _init_l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__4(); -lean_mark_persistent(l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__4); -l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__5 = _init_l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__5(); -lean_mark_persistent(l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__5); -l_Lean_Elab_Command_elabClassInductive___closed__1 = _init_l_Lean_Elab_Command_elabClassInductive___closed__1(); -lean_mark_persistent(l_Lean_Elab_Command_elabClassInductive___closed__1); -l_Lean_Elab_Command_elabClassInductive___closed__2 = _init_l_Lean_Elab_Command_elabClassInductive___closed__2(); -lean_mark_persistent(l_Lean_Elab_Command_elabClassInductive___closed__2); -l_Lean_Elab_Command_elabClassInductive___closed__3 = _init_l_Lean_Elab_Command_elabClassInductive___closed__3(); -lean_mark_persistent(l_Lean_Elab_Command_elabClassInductive___closed__3); l_Lean_Elab_Command_expandNamespacedDeclaration___closed__1 = _init_l_Lean_Elab_Command_expandNamespacedDeclaration___closed__1(); lean_mark_persistent(l_Lean_Elab_Command_expandNamespacedDeclaration___closed__1); l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2 = _init_l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2(); @@ -15842,7 +13614,13 @@ lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1___cl if (builtin) {res = l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Elab_Command_elabInitialize___lambda__1___closed__1 = _init_l_Lean_Elab_Command_elabInitialize___lambda__1___closed__1(); +}l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabInitialize___spec__4___closed__1 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabInitialize___spec__4___closed__1(); +lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabInitialize___spec__4___closed__1); +l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Command_elabInitialize___spec__1___closed__1 = _init_l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Command_elabInitialize___spec__1___closed__1(); +lean_mark_persistent(l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Command_elabInitialize___spec__1___closed__1); +l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Command_elabInitialize___spec__1___closed__2 = _init_l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Command_elabInitialize___spec__1___closed__2(); +lean_mark_persistent(l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Command_elabInitialize___spec__1___closed__2); +l_Lean_Elab_Command_elabInitialize___lambda__1___closed__1 = _init_l_Lean_Elab_Command_elabInitialize___lambda__1___closed__1(); lean_mark_persistent(l_Lean_Elab_Command_elabInitialize___lambda__1___closed__1); l_Lean_Elab_Command_elabInitialize___lambda__1___closed__2 = _init_l_Lean_Elab_Command_elabInitialize___lambda__1___closed__2(); lean_mark_persistent(l_Lean_Elab_Command_elabInitialize___lambda__1___closed__2); @@ -15938,6 +13716,8 @@ l_Lean_Elab_Command_elabInitialize___lambda__1___closed__47 = _init_l_Lean_Elab_ lean_mark_persistent(l_Lean_Elab_Command_elabInitialize___lambda__1___closed__47); l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48 = _init_l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48(); lean_mark_persistent(l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48); +l_Lean_Elab_Command_elabInitialize___lambda__1___closed__49 = _init_l_Lean_Elab_Command_elabInitialize___lambda__1___closed__49(); +lean_mark_persistent(l_Lean_Elab_Command_elabInitialize___lambda__1___closed__49); l_Lean_Elab_Command_elabInitialize___lambda__2___closed__1 = _init_l_Lean_Elab_Command_elabInitialize___lambda__2___closed__1(); lean_mark_persistent(l_Lean_Elab_Command_elabInitialize___lambda__2___closed__1); l_Lean_Elab_Command_elabInitialize___lambda__2___closed__2 = _init_l_Lean_Elab_Command_elabInitialize___lambda__2___closed__2(); @@ -15995,33 +13775,33 @@ lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_elabInitialize__1___closed if (builtin) {res = l___regBuiltin_Lean_Elab_Command_elabInitialize__1(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__1 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__1(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__1); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__2 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__2(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__2); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__3 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__3(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__3); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__4 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__4(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__4); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__5 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__5(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__5); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__6 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__6(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__6); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__7 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__7(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__7); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__8 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__8(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__8); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__9 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__9(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__9); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__10 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__10(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__10); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__11 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__11(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__11); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__12 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__12(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__12); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__13 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__13(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__13); -if (builtin) {res = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024_(lean_io_mk_world()); +}l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__1 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__1(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__1); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__2 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__2(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__2); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__3 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__3(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__3); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__4 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__4(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__4); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__5 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__5(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__5); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__6 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__6(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__6); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__7 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__7(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__7); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__8 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__8(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__8); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__9 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__9(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__9); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__10 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__10(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__10); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__11 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__11(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__11); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__12 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__12(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__12); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__13 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__13(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310____closed__13); +if (builtin) {res = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7310_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }return lean_io_result_mk_ok(lean_box(0)); diff --git a/stage0/stdlib/Lean/Elab/DeclarationRange.c b/stage0/stdlib/Lean/Elab/DeclarationRange.c index 675fa967f956..ac585236cce1 100644 --- a/stage0/stdlib/Lean/Elab/DeclarationRange.c +++ b/stage0/stdlib/Lean/Elab/DeclarationRange.c @@ -13,192 +13,143 @@ #ifdef __cplusplus extern "C" { #endif +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___rarg(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addDeclarationRanges___rarg(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_FileMap_toPosition(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges(lean_object*); -lean_object* l_Lean_Syntax_getPos_x3f(lean_object*, uint8_t); -lean_object* l_Lean_Syntax_getTailPos_x3f(lean_object*, uint8_t); -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___rarg___lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationSelectionRef(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_addDeclarationRanges___rarg___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___rarg___lambda__3(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_addDeclarationRangesForBuiltin___rarg___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___rarg___lambda__1___boxed(lean_object*, lean_object*); uint8_t lean_name_eq(lean_object*, lean_object*); +lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_isIdent(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_FileMap_leanPosToLspPos(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_getDeclarationSelectionRef___closed__2; +static lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___rarg___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___rarg___lambda__1(lean_object*, lean_object*); uint8_t l_Lean_Syntax_isNone(lean_object*); static lean_object* l_Lean_Elab_getDeclarationSelectionRef___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges(lean_object*); -static lean_object* l_Lean_Elab_addDeclarationRanges___rarg___closed__1; +static lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___rarg___lambda__1___closed__1; +lean_object* l_Lean_Syntax_getRange_x3f(lean_object*, uint8_t); +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___rarg___boxed(lean_object*, lean_object*, lean_object*); +lean_object* lean_array_mk(lean_object*); +static lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___rarg___lambda__1___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_getDeclarationSelectionRef___closed__5; -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___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_getDeclarationRange_x3f___rarg___lambda__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_getDeclarationSelectionRef___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin(lean_object*); static lean_object* l_Lean_Elab_getDeclarationSelectionRef___closed__4; -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -uint8_t x_4; lean_object* x_5; lean_object* x_6; -x_4 = 0; -x_5 = l_Lean_Syntax_getPos_x3f(x_1, x_4); -x_6 = l_Lean_Syntax_getTailPos_x3f(x_1, x_4); -if (lean_obj_tag(x_5) == 0) -{ -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_7 = lean_ctor_get(x_2, 0); -lean_inc(x_7); -lean_dec(x_2); -x_8 = lean_ctor_get(x_7, 1); -lean_inc(x_8); -lean_dec(x_7); -x_9 = lean_unsigned_to_nat(0u); +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_4 = lean_ctor_get(x_1, 0); lean_inc(x_3); -x_10 = l_Lean_FileMap_toPosition(x_3, x_9); -lean_inc(x_10); -x_11 = l_Lean_FileMap_leanPosToLspPos(x_3, x_10); -if (lean_obj_tag(x_6) == 0) -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; -lean_dec(x_3); -x_12 = lean_ctor_get(x_11, 1); -lean_inc(x_12); -lean_dec(x_11); -lean_inc(x_12); -lean_inc(x_10); -x_13 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_13, 0, x_10); -lean_ctor_set(x_13, 1, x_12); -lean_ctor_set(x_13, 2, x_10); -lean_ctor_set(x_13, 3, x_12); -x_14 = lean_apply_2(x_8, lean_box(0), x_13); -return x_14; -} -else -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_15 = lean_ctor_get(x_11, 1); -lean_inc(x_15); -lean_dec(x_11); -x_16 = lean_ctor_get(x_6, 0); -lean_inc(x_16); -lean_dec(x_6); +x_5 = l_Lean_FileMap_toPosition(x_3, x_4); +x_6 = lean_ctor_get(x_1, 1); lean_inc(x_3); -x_17 = l_Lean_FileMap_toPosition(x_3, x_16); -lean_dec(x_16); -lean_inc(x_17); -x_18 = l_Lean_FileMap_leanPosToLspPos(x_3, x_17); +x_7 = l_Lean_FileMap_toPosition(x_3, x_6); +x_8 = lean_ctor_get(x_2, 0); +lean_inc(x_8); +lean_dec(x_2); +x_9 = lean_ctor_get(x_8, 1); +lean_inc(x_9); +lean_dec(x_8); +lean_inc(x_5); +x_10 = l_Lean_FileMap_leanPosToLspPos(x_3, x_5); +x_11 = lean_ctor_get(x_10, 1); +lean_inc(x_11); +lean_dec(x_10); +lean_inc(x_7); +x_12 = l_Lean_FileMap_leanPosToLspPos(x_3, x_7); lean_dec(x_3); -x_19 = lean_ctor_get(x_18, 1); -lean_inc(x_19); -lean_dec(x_18); -x_20 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_20, 0, x_10); -lean_ctor_set(x_20, 1, x_15); -lean_ctor_set(x_20, 2, x_17); -lean_ctor_set(x_20, 3, x_19); -x_21 = lean_apply_2(x_8, lean_box(0), x_20); -return x_21; +x_13 = lean_ctor_get(x_12, 1); +lean_inc(x_13); +lean_dec(x_12); +x_14 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_14, 0, x_5); +lean_ctor_set(x_14, 1, x_11); +lean_ctor_set(x_14, 2, x_7); +lean_ctor_set(x_14, 3, x_13); +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_14); +x_16 = lean_apply_2(x_9, lean_box(0), x_15); +return x_16; } } -else +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: { -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_22 = lean_ctor_get(x_2, 0); -lean_inc(x_22); -lean_dec(x_2); -x_23 = lean_ctor_get(x_22, 1); -lean_inc(x_23); -lean_dec(x_22); -x_24 = lean_ctor_get(x_5, 0); -lean_inc(x_24); -lean_dec(x_5); -lean_inc(x_3); -x_25 = l_Lean_FileMap_toPosition(x_3, x_24); -lean_dec(x_24); -lean_inc(x_25); -x_26 = l_Lean_FileMap_leanPosToLspPos(x_3, x_25); -if (lean_obj_tag(x_6) == 0) +uint8_t x_4; lean_object* x_5; +x_4 = 0; +x_5 = l_Lean_Syntax_getRange_x3f(x_3, x_4); +if (lean_obj_tag(x_5) == 0) { -lean_object* x_27; lean_object* x_28; lean_object* x_29; -lean_dec(x_3); -x_27 = lean_ctor_get(x_26, 1); -lean_inc(x_27); -lean_dec(x_26); -lean_inc(x_27); -lean_inc(x_25); -x_28 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_28, 0, x_25); -lean_ctor_set(x_28, 1, x_27); -lean_ctor_set(x_28, 2, x_25); -lean_ctor_set(x_28, 3, x_27); -x_29 = lean_apply_2(x_23, lean_box(0), x_28); -return x_29; +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_dec(x_2); +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +lean_dec(x_1); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +x_8 = lean_box(0); +x_9 = lean_apply_2(x_7, lean_box(0), x_8); +return x_9; } else { -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_30 = lean_ctor_get(x_26, 1); -lean_inc(x_30); -lean_dec(x_26); -x_31 = lean_ctor_get(x_6, 0); -lean_inc(x_31); -lean_dec(x_6); -lean_inc(x_3); -x_32 = l_Lean_FileMap_toPosition(x_3, x_31); -lean_dec(x_31); -lean_inc(x_32); -x_33 = l_Lean_FileMap_leanPosToLspPos(x_3, x_32); -lean_dec(x_3); -x_34 = lean_ctor_get(x_33, 1); -lean_inc(x_34); -lean_dec(x_33); -x_35 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_35, 0, x_25); -lean_ctor_set(x_35, 1, x_30); -lean_ctor_set(x_35, 2, x_32); -lean_ctor_set(x_35, 3, x_34); -x_36 = lean_apply_2(x_23, lean_box(0), x_35); -return x_36; -} +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_Lean_Elab_getDeclarationRange_x3f___rarg___lambda__1___boxed), 3, 2); +lean_closure_set(x_12, 0, x_10); +lean_closure_set(x_12, 1, x_1); +x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_2, x_12); +return x_13; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f(lean_object* x_1) { _start: { -lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_4 = lean_ctor_get(x_1, 1); -lean_inc(x_4); -x_5 = lean_alloc_closure((void*)(l_Lean_Elab_getDeclarationRange___rarg___lambda__1___boxed), 3, 2); -lean_closure_set(x_5, 0, x_3); -lean_closure_set(x_5, 1, x_1); -x_6 = lean_apply_4(x_4, lean_box(0), lean_box(0), x_2, x_5); -return x_6; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Elab_getDeclarationRange_x3f___rarg___boxed), 3, 0); +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Elab_getDeclarationRange___rarg), 3, 0); -return x_2; +lean_object* x_4; +x_4 = l_Lean_Elab_getDeclarationRange_x3f___rarg___lambda__1(x_1, x_2, x_3); +lean_dec(x_1); +return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Lean_Elab_getDeclarationRange___rarg___lambda__1(x_1, x_2, x_3); -lean_dec(x_1); +x_4 = l_Lean_Elab_getDeclarationRange_x3f___rarg(x_1, x_2, x_3); +lean_dec(x_3); return x_4; } } @@ -314,7 +265,24 @@ return x_17; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___rarg___lambda__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +lean_inc(x_1); +return x_1; +} +else +{ +lean_object* x_3; +x_3 = lean_ctor_get(x_2, 0); +lean_inc(x_3); +return x_3; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___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; @@ -325,142 +293,242 @@ x_7 = l_Lean_addDeclarationRanges___rarg(x_2, x_3, x_4, x_6); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___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: { +if (lean_obj_tag(x_7) == 0) +{ lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_8 = l_Lean_Elab_getDeclarationSelectionRef(x_1); -lean_inc(x_2); -x_9 = l_Lean_Elab_getDeclarationRange___rarg(x_2, x_3, x_8); -x_10 = lean_alloc_closure((void*)(l_Lean_Elab_addDeclarationRanges___rarg___lambda__1), 5, 4); -lean_closure_set(x_10, 0, x_7); -lean_closure_set(x_10, 1, x_2); -lean_closure_set(x_10, 2, x_4); -lean_closure_set(x_10, 3, x_5); -x_11 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_9, x_10); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +x_8 = lean_ctor_get(x_1, 0); +lean_inc(x_8); +lean_dec(x_1); +x_9 = lean_ctor_get(x_8, 1); +lean_inc(x_9); +lean_dec(x_8); +x_10 = lean_box(0); +x_11 = lean_apply_2(x_9, lean_box(0), x_10); return x_11; } +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_12 = lean_ctor_get(x_7, 0); +lean_inc(x_12); +lean_dec(x_7); +x_13 = lean_ctor_get(x_1, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +lean_dec(x_13); +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +lean_dec(x_14); +lean_inc(x_12); +x_16 = lean_alloc_closure((void*)(l_Lean_Elab_addDeclarationRangesFromSyntax___rarg___lambda__1___boxed), 2, 1); +lean_closure_set(x_16, 0, x_12); +lean_inc(x_1); +x_17 = l_Lean_Elab_getDeclarationRange_x3f___rarg(x_1, x_2, x_3); +x_18 = lean_apply_4(x_15, lean_box(0), lean_box(0), x_16, x_17); +x_19 = lean_alloc_closure((void*)(l_Lean_Elab_addDeclarationRangesFromSyntax___rarg___lambda__2), 5, 4); +lean_closure_set(x_19, 0, x_12); +lean_closure_set(x_19, 1, x_1); +lean_closure_set(x_19, 2, x_4); +lean_closure_set(x_19, 3, x_5); +x_20 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_18, x_19); +return x_20; +} } -static lean_object* _init_l_Lean_Elab_addDeclarationRanges___rarg___closed__1() { +} +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___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_1; -x_1 = lean_mk_string_unchecked("example", 7, 7); -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_1, 1); +lean_inc(x_7); +lean_inc(x_3); +lean_inc(x_1); +x_8 = l_Lean_Elab_getDeclarationRange_x3f___rarg(x_1, x_3, x_5); +lean_inc(x_7); +x_9 = lean_alloc_closure((void*)(l_Lean_Elab_addDeclarationRangesFromSyntax___rarg___lambda__3___boxed), 7, 6); +lean_closure_set(x_9, 0, x_1); +lean_closure_set(x_9, 1, x_3); +lean_closure_set(x_9, 2, x_6); +lean_closure_set(x_9, 3, x_2); +lean_closure_set(x_9, 4, x_4); +lean_closure_set(x_9, 5, x_7); +x_10 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_8, x_9); +return x_10; } } -static lean_object* _init_l_Lean_Elab_addDeclarationRanges___rarg___closed__2() { +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax(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_Elab_getDeclarationSelectionRef___closed__1; -x_2 = l_Lean_Elab_getDeclarationSelectionRef___closed__2; -x_3 = l_Lean_Elab_getDeclarationSelectionRef___closed__3; -x_4 = l_Lean_Elab_addDeclarationRanges___rarg___closed__1; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Elab_addDeclarationRangesFromSyntax___rarg___boxed), 6, 0); +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_6; lean_object* x_7; uint8_t x_8; -lean_inc(x_5); -x_6 = l_Lean_Syntax_getKind(x_5); -x_7 = l_Lean_Elab_addDeclarationRanges___rarg___closed__2; -x_8 = lean_name_eq(x_6, x_7); -lean_dec(x_6); -if (x_8 == 0) +lean_object* x_3; +x_3 = l_Lean_Elab_addDeclarationRangesFromSyntax___rarg___lambda__1(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___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; lean_object* x_11; lean_object* x_12; -x_9 = lean_ctor_get(x_1, 1); -lean_inc(x_9); -lean_inc(x_5); -lean_inc(x_3); -lean_inc(x_1); -x_10 = l_Lean_Elab_getDeclarationRange___rarg(x_1, x_3, x_5); -lean_inc(x_9); -x_11 = lean_alloc_closure((void*)(l_Lean_Elab_addDeclarationRanges___rarg___lambda__2), 7, 6); -lean_closure_set(x_11, 0, x_5); -lean_closure_set(x_11, 1, x_1); -lean_closure_set(x_11, 2, x_3); -lean_closure_set(x_11, 3, x_2); -lean_closure_set(x_11, 4, x_4); -lean_closure_set(x_11, 5, x_9); -x_12 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_10, x_11); -return x_12; +lean_object* x_8; +x_8 = l_Lean_Elab_addDeclarationRangesFromSyntax___rarg___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_3); +return x_8; } -else +} +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +lean_object* x_7; +x_7 = l_Lean_Elab_addDeclarationRangesFromSyntax___rarg(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_13 = lean_ctor_get(x_1, 0); -lean_inc(x_13); -lean_dec(x_1); -x_14 = lean_ctor_get(x_13, 1); -lean_inc(x_14); -lean_dec(x_13); -x_15 = lean_box(0); -x_16 = lean_apply_2(x_14, lean_box(0), x_15); -return x_16; +return x_7; +} } +static lean_object* _init_l_Lean_Elab_addDeclarationRangesForBuiltin___rarg___lambda__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("null", 4, 4); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges(lean_object* x_1) { +static lean_object* _init_l_Lean_Elab_addDeclarationRangesForBuiltin___rarg___lambda__1___closed__2() { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Elab_addDeclarationRanges___rarg), 5, 0); -return x_2; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_addDeclarationRangesForBuiltin___rarg___lambda__1___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { -lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_8 = lean_box(0); lean_inc(x_1); -x_8 = l_Lean_Elab_getDeclarationRange___rarg(x_1, x_2, x_3); -x_9 = lean_alloc_closure((void*)(l_Lean_Elab_addDeclarationRanges___rarg___lambda__1), 5, 4); -lean_closure_set(x_9, 0, x_7); -lean_closure_set(x_9, 1, x_1); -lean_closure_set(x_9, 2, x_4); -lean_closure_set(x_9, 3, x_5); -x_10 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_8, x_9); -return x_10; +x_9 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_9, 0, x_1); +lean_ctor_set(x_9, 1, x_8); +x_10 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_10, 0, x_2); +lean_ctor_set(x_10, 1, x_9); +x_11 = lean_array_mk(x_10); +x_12 = lean_box(2); +x_13 = l_Lean_Elab_addDeclarationRangesForBuiltin___rarg___lambda__1___closed__2; +x_14 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_14, 0, x_12); +lean_ctor_set(x_14, 1, x_13); +lean_ctor_set(x_14, 2, x_11); +x_15 = l_Lean_Elab_getDeclarationSelectionRef(x_1); +x_16 = l_Lean_Elab_addDeclarationRangesFromSyntax___rarg(x_3, x_4, x_5, x_6, x_14, x_15); +lean_dec(x_14); +return x_16; } } -LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +static lean_object* _init_l_Lean_Elab_addDeclarationRangesForBuiltin___rarg___closed__1() { _start: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; -x_7 = lean_ctor_get(x_1, 1); -lean_inc(x_7); -lean_inc(x_3); +lean_object* x_1; +x_1 = lean_mk_string_unchecked("example", 7, 7); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_addDeclarationRangesForBuiltin___rarg___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_Elab_getDeclarationSelectionRef___closed__1; +x_2 = l_Lean_Elab_getDeclarationSelectionRef___closed__2; +x_3 = l_Lean_Elab_getDeclarationSelectionRef___closed__3; +x_4 = l_Lean_Elab_addDeclarationRangesForBuiltin___rarg___closed__1; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___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; lean_inc(x_1); -x_8 = l_Lean_Elab_getDeclarationRange___rarg(x_1, x_3, x_5); -lean_inc(x_7); -x_9 = lean_alloc_closure((void*)(l_Lean_Elab_addAuxDeclarationRanges___rarg___lambda__1), 7, 6); -lean_closure_set(x_9, 0, x_1); -lean_closure_set(x_9, 1, x_3); -lean_closure_set(x_9, 2, x_6); -lean_closure_set(x_9, 3, x_2); -lean_closure_set(x_9, 4, x_4); -lean_closure_set(x_9, 5, x_7); -x_10 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_8, x_9); -return x_10; +lean_inc(x_6); +x_7 = lean_alloc_closure((void*)(l_Lean_Elab_addDeclarationRangesForBuiltin___rarg___lambda__1___boxed), 7, 6); +lean_closure_set(x_7, 0, x_6); +lean_closure_set(x_7, 1, x_5); +lean_closure_set(x_7, 2, x_1); +lean_closure_set(x_7, 3, x_2); +lean_closure_set(x_7, 4, x_3); +lean_closure_set(x_7, 5, x_4); +x_8 = l_Lean_Syntax_getKind(x_6); +x_9 = l_Lean_Elab_addDeclarationRangesForBuiltin___rarg___closed__2; +x_10 = lean_name_eq(x_8, x_9); +lean_dec(x_8); +if (x_10 == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_11 = lean_ctor_get(x_1, 1); +lean_inc(x_11); +x_12 = lean_ctor_get(x_1, 0); +lean_inc(x_12); +lean_dec(x_1); +x_13 = lean_ctor_get(x_12, 1); +lean_inc(x_13); +lean_dec(x_12); +x_14 = lean_box(0); +x_15 = lean_apply_2(x_13, lean_box(0), x_14); +x_16 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_15, x_7); +return x_16; +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +lean_dec(x_7); +x_17 = lean_ctor_get(x_1, 0); +lean_inc(x_17); +lean_dec(x_1); +x_18 = lean_ctor_get(x_17, 1); +lean_inc(x_18); +lean_dec(x_17); +x_19 = lean_box(0); +x_20 = lean_apply_2(x_18, lean_box(0), x_19); +return x_20; } } -LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges(lean_object* x_1) { +} +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Elab_addAuxDeclarationRanges___rarg), 6, 0); +x_2 = lean_alloc_closure((void*)(l_Lean_Elab_addDeclarationRangesForBuiltin___rarg), 6, 0); return x_2; } } +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; +x_8 = l_Lean_Elab_addDeclarationRangesForBuiltin___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_7); +return x_8; +} +} lean_object* initialize_Lean_Log(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Parser_Command(uint8_t builtin, lean_object*); lean_object* initialize_Lean_DeclarationRange(uint8_t builtin, lean_object*); @@ -492,10 +560,14 @@ l_Lean_Elab_getDeclarationSelectionRef___closed__4 = _init_l_Lean_Elab_getDeclar lean_mark_persistent(l_Lean_Elab_getDeclarationSelectionRef___closed__4); l_Lean_Elab_getDeclarationSelectionRef___closed__5 = _init_l_Lean_Elab_getDeclarationSelectionRef___closed__5(); lean_mark_persistent(l_Lean_Elab_getDeclarationSelectionRef___closed__5); -l_Lean_Elab_addDeclarationRanges___rarg___closed__1 = _init_l_Lean_Elab_addDeclarationRanges___rarg___closed__1(); -lean_mark_persistent(l_Lean_Elab_addDeclarationRanges___rarg___closed__1); -l_Lean_Elab_addDeclarationRanges___rarg___closed__2 = _init_l_Lean_Elab_addDeclarationRanges___rarg___closed__2(); -lean_mark_persistent(l_Lean_Elab_addDeclarationRanges___rarg___closed__2); +l_Lean_Elab_addDeclarationRangesForBuiltin___rarg___lambda__1___closed__1 = _init_l_Lean_Elab_addDeclarationRangesForBuiltin___rarg___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Elab_addDeclarationRangesForBuiltin___rarg___lambda__1___closed__1); +l_Lean_Elab_addDeclarationRangesForBuiltin___rarg___lambda__1___closed__2 = _init_l_Lean_Elab_addDeclarationRangesForBuiltin___rarg___lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Elab_addDeclarationRangesForBuiltin___rarg___lambda__1___closed__2); +l_Lean_Elab_addDeclarationRangesForBuiltin___rarg___closed__1 = _init_l_Lean_Elab_addDeclarationRangesForBuiltin___rarg___closed__1(); +lean_mark_persistent(l_Lean_Elab_addDeclarationRangesForBuiltin___rarg___closed__1); +l_Lean_Elab_addDeclarationRangesForBuiltin___rarg___closed__2 = _init_l_Lean_Elab_addDeclarationRangesForBuiltin___rarg___closed__2(); +lean_mark_persistent(l_Lean_Elab_addDeclarationRangesForBuiltin___rarg___closed__2); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Lean/Elab/DefView.c b/stage0/stdlib/Lean/Elab/DefView.c index fdefcf32ea6c..2d58b955f865 100644 --- a/stage0/stdlib/Lean/Elab/DefView.c +++ b/stage0/stdlib/Lean/Elab/DefView.c @@ -1005,20 +1005,22 @@ return x_6; static lean_object* _init_l_Lean_Elab_instInhabitedDefView___closed__1() { _start: { -lean_object* x_1; uint8_t x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; +lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; uint8_t x_5; lean_object* x_6; lean_object* x_7; x_1 = lean_box(0); -x_2 = 0; +x_2 = lean_box(0); x_3 = 0; x_4 = 0; -x_5 = l_Lean_Elab_instInhabitedDefViewElabHeaderData___closed__1; -x_6 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_6, 0, x_1); -lean_ctor_set(x_6, 1, x_5); -lean_ctor_set_uint8(x_6, sizeof(void*)*2, x_2); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 1, x_3); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 2, x_4); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 3, x_3); -return x_6; +x_5 = 0; +x_6 = l_Lean_Elab_instInhabitedDefViewElabHeaderData___closed__1; +x_7 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_7, 0, x_2); +lean_ctor_set(x_7, 1, x_1); +lean_ctor_set(x_7, 2, x_6); +lean_ctor_set_uint8(x_7, sizeof(void*)*3, x_3); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 1, x_4); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 2, x_5); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 3, x_4); +return x_7; } } static lean_object* _init_l_Lean_Elab_instInhabitedDefView___closed__2() { @@ -1112,7 +1114,7 @@ LEAN_EXPORT uint8_t l_Lean_Elab_DefView_isInstance(lean_object* x_1) { { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; uint8_t x_6; x_2 = lean_ctor_get(x_1, 2); -x_3 = lean_ctor_get(x_2, 1); +x_3 = lean_ctor_get(x_2, 2); x_4 = lean_array_get_size(x_3); x_5 = lean_unsigned_to_nat(0u); x_6 = lean_nat_dec_lt(x_5, x_4); @@ -4899,7 +4901,7 @@ uint8_t x_15; lean_dec(x_10); lean_dec(x_9); lean_dec(x_2); -x_15 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 3); +x_15 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 3); lean_dec(x_1); if (x_15 == 0) { diff --git a/stage0/stdlib/Lean/Elab/Deriving/BEq.c b/stage0/stdlib/Lean/Elab/Deriving/BEq.c index a79141855c09..b4fea22d10c5 100644 --- a/stage0/stdlib/Lean/Elab/Deriving/BEq.c +++ b/stage0/stdlib/Lean/Elab/Deriving/BEq.c @@ -14,7 +14,6 @@ extern "C" { #endif static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_BEq_mkMatch_mkAlts___spec__5___lambda__1___closed__12; -LEAN_EXPORT lean_object* l_List_allM___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_getConstInfoCtor___at_Lean_Elab_Deriving_BEq_mkMatch_mkAlts___spec__1___closed__3; lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_BEq_mkMatch_mkAlts___spec__5___lambda__1___closed__34; @@ -23,6 +22,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_BEq_mkAuxFunction___lambda__1(lean static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_BEq_mkMatch_mkAlts___spec__5___lambda__1___closed__39; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Deriving_BEq_mkBEqInstanceHandler___spec__3(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_BEq_mkMatch_mkAlts___spec__5___lambda__1___closed__17; +static lean_object* l_Lean_getConstInfo___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__2___closed__1; static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_BEq_mkMatch_mkAlts___spec__7___lambda__1___closed__8; static lean_object* l_Lean_Elab_Deriving_BEq_mkAuxFunction___lambda__1___closed__22; static lean_object* l_Lean_Elab_Deriving_BEq_mkAuxFunction___lambda__1___closed__2; @@ -33,10 +33,12 @@ static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_BEq_mkMatch_mkAlts static lean_object* l_Lean_Elab_Deriving_BEq_mkMatch_mkElseAlt___closed__13; static lean_object* l_Lean_Elab_Deriving_BEq_mkMutualBlock___closed__4; LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_BEq_mkMutualBlock___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_BEq_mkMatch_mkAlts___spec__5___lambda__1___closed__25; static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_BEq_mkMatch_mkAlts___spec__5___lambda__1___closed__28; static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_BEq_mkMatch_mkAlts___spec__5___lambda__1___closed__7; static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_BEq_mkMatch_mkAlts___spec__5___closed__1; +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__3___boxed(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_Deriving_BEq_mkAuxFunction___lambda__1___closed__7; static lean_object* l_Lean_Elab_Deriving_BEq_mkMatch_mkElseAlt___closed__16; @@ -75,6 +77,7 @@ lean_object* l_Lean_Elab_Deriving_mkLocalInstanceLetDecls(lean_object*, lean_obj uint8_t l_Lean_Expr_isAppOf(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Deriving_BEq_0__Lean_Elab_Deriving_BEq_mkBEqEnumFun___closed__11; static lean_object* l_Lean_Elab_Deriving_BEq_mkAuxFunction___lambda__1___closed__19; +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_node5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_stringToMessageData(lean_object*); static lean_object* l___private_Lean_Elab_Deriving_BEq_0__Lean_Elab_Deriving_BEq_mkBEqEnumFun___closed__7; @@ -106,7 +109,6 @@ static lean_object* l_Lean_Elab_Deriving_BEq_mkAuxFunction___lambda__1___closed_ lean_object* l_Array_reverse___rarg(lean_object*); lean_object* l_Lean_Elab_registerDerivingHandler(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_BEq_mkMatch_mkElseAlt___closed__12; -lean_object* l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Deriving_BEq_0__Lean_Elab_Deriving_BEq_mkBEqEnumFun___closed__9; lean_object* l_Lean_Elab_Deriving_mkLet(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Deriving_BEq_0__Lean_Elab_Deriving_BEq_mkBEqInstanceCmds___closed__6; @@ -124,6 +126,7 @@ static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_BEq_mkMatch_m lean_object* l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_BEq_mkMatch_mkAlts___spec__7___lambda__1___closed__3; lean_object* l_Lean_registerTraceClass(lean_object*, uint8_t, lean_object*, lean_object*); +lean_object* l_Lean_Elab_Command_getRef(lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_CoreM_0__Lean_Core_mkFreshNameImp(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getConstInfoCtor___at_Lean_Elab_Deriving_BEq_mkMatch_mkAlts___spec__1___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_Lean_Elab_Deriving_BEq_mkMatch_mkAlts___spec__5___lambda__1___closed__21; @@ -175,6 +178,7 @@ static lean_object* l_Lean_Elab_Deriving_BEq_mkMatch_mkElseAlt___closed__17; static lean_object* l_Lean_Elab_Deriving_BEq_initFn____x40_Lean_Elab_Deriving_BEq___hyg_3922____closed__16; lean_object* l_Lean_Syntax_node2(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_BEq_mkMatch_mkAlts___spec__5___lambda__1___closed__9; +lean_object* l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_BEq_mkMatch_mkElseAlt(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_BEq_mkMatch___closed__4; static lean_object* l_Lean_Elab_Deriving_BEq_mkBEqHeader___closed__1; @@ -221,9 +225,11 @@ static lean_object* l_Lean_Elab_Deriving_BEq_mkMutualBlock___closed__11; static lean_object* l_Lean_Elab_Deriving_BEq_mkAuxFunction___lambda__1___closed__4; static lean_object* l_Lean_Elab_Deriving_BEq_mkAuxFunction___lambda__1___closed__11; static lean_object* l_Lean_Elab_Deriving_BEq_mkMutualBlock___closed__1; +static lean_object* l_Lean_getConstInfo___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__2___closed__2; static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_BEq_mkMatch_mkAlts___spec__5___lambda__1___closed__14; LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_BEq_mkBEqInstance(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_BEq_mkAuxFunction___lambda__1___closed__25; +LEAN_EXPORT lean_object* l_List_allM___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_BEq_mkAuxFunction___lambda__1___closed__15; lean_object* l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); @@ -232,6 +238,7 @@ static lean_object* l_Lean_Elab_Deriving_BEq_mkAuxFunction___lambda__1___closed_ uint8_t lean_nat_dec_lt(lean_object*, lean_object*); lean_object* lean_environment_main_module(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Deriving_BEq_mkBEqInstanceHandler___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_allM___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_isEnumType___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_BEq_mkMatch_mkAlts___spec__5___lambda__1___closed__20; @@ -254,7 +261,6 @@ lean_object* l_Lean_Meta_forallTelescopeReducing___at_Lean_Elab_Deriving_mkInduc static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_BEq_mkMatch_mkAlts___spec__5___closed__3; lean_object* l_Array_mkArray1___rarg(lean_object*); uint8_t l_Lean_Expr_isProp(lean_object*); -LEAN_EXPORT lean_object* l_List_allM___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_BEq_mkAuxFunction___lambda__1___closed__12; static lean_object* l_Lean_Elab_Deriving_BEq_initFn____x40_Lean_Elab_Deriving_BEq___hyg_3922____closed__6; static lean_object* l_Lean_Elab_Deriving_BEq_initFn____x40_Lean_Elab_Deriving_BEq___hyg_3922____closed__12; @@ -276,6 +282,7 @@ size_t lean_usize_add(size_t, size_t); static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_BEq_mkMatch_mkAlts___spec__5___closed__4; static lean_object* l_Lean_Elab_Deriving_BEq_initFn____x40_Lean_Elab_Deriving_BEq___hyg_3922____closed__4; lean_object* l_Lean_Syntax_node8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_instInhabitedName; static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_BEq_mkMatch_mkElseAlt___spec__1___closed__4; lean_object* lean_array_uget(lean_object*, size_t); @@ -287,6 +294,7 @@ LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_BEq_mkMatch_m extern lean_object* l_Lean_instInhabitedInductiveVal; static lean_object* l_Lean_Elab_Deriving_BEq_mkAuxFunction___lambda__1___closed__8; lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_BEq_initFn____x40_Lean_Elab_Deriving_BEq___hyg_3922____closed__1; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Deriving_BEq_mkMatch_mkAlts___spec__4(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_BEq_mkMatch_mkAlts___spec__5___lambda__1___closed__42; @@ -8903,7 +8911,204 @@ return x_91; } } } -LEAN_EXPORT lean_object* l_List_allM___at_Lean_Elab_Deriving_BEq_mkBEqInstance___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_Elab_Deriving_BEq_mkBEqInstance___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_5 = l_Lean_Elab_Command_getRef(x_2, x_3, x_4); +x_6 = lean_ctor_get(x_5, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_5, 1); +lean_inc(x_7); +lean_dec(x_5); +x_8 = lean_ctor_get(x_2, 4); +lean_inc(x_8); +lean_inc(x_8); +x_9 = l_Lean_Elab_getBetterRef(x_6, x_8); +lean_dec(x_6); +x_10 = l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1(x_1, x_2, x_3, x_7); +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_12 = lean_ctor_get(x_10, 0); +x_13 = lean_ctor_get(x_10, 1); +x_14 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_12, x_8, x_2, x_3, x_13); +lean_dec(x_2); +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 0) +{ +lean_object* x_16; +x_16 = lean_ctor_get(x_14, 0); +lean_ctor_set(x_10, 1, x_16); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set_tag(x_14, 1); +lean_ctor_set(x_14, 0, x_10); +return x_14; +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_14, 0); +x_18 = lean_ctor_get(x_14, 1); +lean_inc(x_18); +lean_inc(x_17); +lean_dec(x_14); +lean_ctor_set(x_10, 1, x_17); +lean_ctor_set(x_10, 0, x_9); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_10); +lean_ctor_set(x_19, 1, 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; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_20 = lean_ctor_get(x_10, 0); +x_21 = lean_ctor_get(x_10, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_10); +x_22 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_20, x_8, x_2, x_3, x_21); +lean_dec(x_2); +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +if (lean_is_exclusive(x_22)) { + lean_ctor_release(x_22, 0); + lean_ctor_release(x_22, 1); + x_25 = x_22; +} else { + lean_dec_ref(x_22); + x_25 = lean_box(0); +} +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_9); +lean_ctor_set(x_26, 1, x_23); +if (lean_is_scalar(x_25)) { + x_27 = lean_alloc_ctor(1, 2, 0); +} else { + x_27 = x_25; + lean_ctor_set_tag(x_27, 1); +} +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_24); +return x_27; +} +} +} +static lean_object* _init_l_Lean_getConstInfo___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__2___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("unknown constant '", 18, 18); +return x_1; +} +} +static lean_object* _init_l_Lean_getConstInfo___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__2___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_getConstInfo___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__2___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; uint8_t x_6; +x_5 = lean_st_ref_get(x_3, x_4); +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; +x_7 = lean_ctor_get(x_5, 0); +x_8 = lean_ctor_get(x_5, 1); +x_9 = lean_ctor_get(x_7, 0); +lean_inc(x_9); +lean_dec(x_7); +lean_inc(x_1); +x_10 = lean_environment_find(x_9, x_1); +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; +lean_free_object(x_5); +x_11 = lean_box(0); +x_12 = l_Lean_Expr_const___override(x_1, x_11); +x_13 = l_Lean_MessageData_ofExpr(x_12); +x_14 = l_Lean_getConstInfo___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__2___closed__2; +x_15 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_13); +x_16 = l_Lean_getConstInfoCtor___at_Lean_Elab_Deriving_BEq_mkMatch_mkAlts___spec__1___closed__2; +x_17 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_17, 0, x_15); +lean_ctor_set(x_17, 1, x_16); +x_18 = l_Lean_throwError___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__3(x_17, x_2, x_3, x_8); +return x_18; +} +else +{ +lean_object* x_19; +lean_dec(x_2); +lean_dec(x_1); +x_19 = lean_ctor_get(x_10, 0); +lean_inc(x_19); +lean_dec(x_10); +lean_ctor_set(x_5, 0, x_19); +return x_5; +} +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_20 = lean_ctor_get(x_5, 0); +x_21 = lean_ctor_get(x_5, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_5); +x_22 = lean_ctor_get(x_20, 0); +lean_inc(x_22); +lean_dec(x_20); +lean_inc(x_1); +x_23 = lean_environment_find(x_22, x_1); +if (lean_obj_tag(x_23) == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_24 = lean_box(0); +x_25 = l_Lean_Expr_const___override(x_1, x_24); +x_26 = l_Lean_MessageData_ofExpr(x_25); +x_27 = l_Lean_getConstInfo___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__2___closed__2; +x_28 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_26); +x_29 = l_Lean_getConstInfoCtor___at_Lean_Elab_Deriving_BEq_mkMatch_mkAlts___spec__1___closed__2; +x_30 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +x_31 = l_Lean_throwError___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__3(x_30, x_2, x_3, x_21); +return x_31; +} +else +{ +lean_object* x_32; lean_object* x_33; +lean_dec(x_2); +lean_dec(x_1); +x_32 = lean_ctor_get(x_23, 0); +lean_inc(x_32); +lean_dec(x_23); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_21); +return x_33; +} +} +} +} +LEAN_EXPORT lean_object* l_List_allM___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { if (lean_obj_tag(x_1) == 0) @@ -8933,7 +9138,7 @@ if (lean_is_exclusive(x_1)) { x_10 = lean_box(0); } lean_inc(x_2); -x_18 = l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9(x_8, x_2, x_3, x_4); +x_18 = l_Lean_getConstInfo___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__2(x_8, x_2, x_3, x_4); if (lean_obj_tag(x_18) == 0) { lean_object* x_19; @@ -9031,7 +9236,7 @@ LEAN_EXPORT lean_object* l_Lean_isEnumType___at_Lean_Elab_Deriving_BEq_mkBEqInst { lean_object* x_5; lean_inc(x_2); -x_5 = l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9(x_1, x_2, x_3, x_4); +x_5 = l_Lean_getConstInfo___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__2(x_1, x_2, x_3, x_4); if (lean_obj_tag(x_5) == 0) { lean_object* x_6; @@ -9128,7 +9333,7 @@ if (x_31 == 0) { lean_object* x_32; lean_free_object(x_5); -x_32 = l_List_allM___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__2(x_28, x_2, x_3, x_8); +x_32 = l_List_allM___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__4(x_28, x_2, x_3, x_8); return x_32; } else @@ -9272,7 +9477,7 @@ lean_dec(x_42); if (x_66 == 0) { lean_object* x_67; -x_67 = l_List_allM___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__2(x_63, x_2, x_3, x_41); +x_67 = l_List_allM___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__4(x_63, x_2, x_3, x_41); return x_67; } else @@ -9713,11 +9918,29 @@ return x_79; } } } -LEAN_EXPORT lean_object* l_List_allM___at_Lean_Elab_Deriving_BEq_mkBEqInstance___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_Elab_Deriving_BEq_mkBEqInstance___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Lean_throwError___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__3(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at_Lean_Elab_Deriving_BEq_mkBEqInstance___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_getConstInfo___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__2(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_List_allM___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_List_allM___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__2(x_1, x_2, x_3, x_4); +x_5 = l_List_allM___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__4(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } @@ -10670,6 +10893,10 @@ l___private_Lean_Elab_Deriving_BEq_0__Lean_Elab_Deriving_BEq_mkBEqEnumFun___clos lean_mark_persistent(l___private_Lean_Elab_Deriving_BEq_0__Lean_Elab_Deriving_BEq_mkBEqEnumFun___closed__16); l___private_Lean_Elab_Deriving_BEq_0__Lean_Elab_Deriving_BEq_mkBEqEnumFun___closed__17 = _init_l___private_Lean_Elab_Deriving_BEq_0__Lean_Elab_Deriving_BEq_mkBEqEnumFun___closed__17(); lean_mark_persistent(l___private_Lean_Elab_Deriving_BEq_0__Lean_Elab_Deriving_BEq_mkBEqEnumFun___closed__17); +l_Lean_getConstInfo___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__2___closed__1 = _init_l_Lean_getConstInfo___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__2___closed__1(); +lean_mark_persistent(l_Lean_getConstInfo___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__2___closed__1); +l_Lean_getConstInfo___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__2___closed__2 = _init_l_Lean_getConstInfo___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__2___closed__2(); +lean_mark_persistent(l_Lean_getConstInfo___at_Lean_Elab_Deriving_BEq_mkBEqInstance___spec__2___closed__2); l_Lean_Elab_Deriving_BEq_initFn____x40_Lean_Elab_Deriving_BEq___hyg_3922____closed__1 = _init_l_Lean_Elab_Deriving_BEq_initFn____x40_Lean_Elab_Deriving_BEq___hyg_3922____closed__1(); lean_mark_persistent(l_Lean_Elab_Deriving_BEq_initFn____x40_Lean_Elab_Deriving_BEq___hyg_3922____closed__1); l_Lean_Elab_Deriving_BEq_initFn____x40_Lean_Elab_Deriving_BEq___hyg_3922____closed__2 = _init_l_Lean_Elab_Deriving_BEq_initFn____x40_Lean_Elab_Deriving_BEq___hyg_3922____closed__2(); diff --git a/stage0/stdlib/Lean/Elab/Deriving/DecEq.c b/stage0/stdlib/Lean/Elab/Deriving/DecEq.c index f41b3a99daca..b8c939b62d5b 100644 --- a/stage0/stdlib/Lean/Elab/Deriving/DecEq.c +++ b/stage0/stdlib/Lean/Elab/Deriving/DecEq.c @@ -15,7 +15,6 @@ extern "C" { #endif static lean_object* l_Lean_getConstInfoCtor___at_Lean_Elab_Deriving_DecEq_mkMatch_mkAlts___spec__1___closed__1; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_DecEq_mkMatch_mkAlts___spec__6___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_DecEq_mkEnumOfNat_mkDecTree___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEq___lambda__1(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); @@ -48,6 +47,7 @@ static lean_object* l_Lean_Elab_Deriving_DecEq_mkAuxFunction___lambda__1___close static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__3___closed__4; 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__5; +LEAN_EXPORT lean_object* l_Lean_Elab_enableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEqEnum___closed__4; lean_object* l_Lean_Meta_isProp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEqEnum___closed__16; @@ -85,9 +85,10 @@ static lean_object* l_Lean_Elab_Deriving_DecEq_mkAuxFunction___closed__5; static lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEqEnum___closed__17; LEAN_EXPORT lean_object* l_Lean_isEnumType___at_Lean_Elab_Deriving_DecEq_mkDecEqInstance___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_fvarId_x21(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_enableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__4(uint8_t, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEqEnum___closed__41; +lean_object* lean_environment_find(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEqEnum___closed__9; +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_DecEq_mkEnumOfNat_mkDecTree___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___closed__6; @@ -125,9 +126,7 @@ lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec static lean_object* l_Lean_Elab_Deriving_DecEq_mkEnumOfNat___lambda__1___closed__1; static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__2___closed__51; static lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEqCmds___closed__5; -LEAN_EXPORT lean_object* l_Lean_Elab_withEnableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__3(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_DecEq_initFn____x40_Lean_Elab_Deriving_DecEq___hyg_4874____closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_withEnableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_mapMUnsafe_map___at___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___spec__3(size_t, size_t, lean_object*); static lean_object* l_Lean_Elab_Deriving_DecEq_mkAuxFunction___lambda__1___closed__7; static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___closed__4; @@ -142,13 +141,13 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEqCmds(lean_object*, le size_t lean_usize_of_nat(lean_object*); static lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEqEnum___closed__28; static lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEqEnum___closed__49; +static lean_object* l_Lean_getConstInfo___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__2___closed__1; static lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEqEnum___closed__10; 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*); static lean_object* l_Lean_Elab_Deriving_DecEq_mkEnumOfNat___closed__2; LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_Deriving_DecEq_mkDecEqCmds___spec__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__2___closed__29; lean_object* l_Lean_Elab_registerDerivingHandler(lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_DecEq_mkMatch_mkAlts___spec__6___closed__1; lean_object* lean_st_ref_take(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_DecEq_mkAuxFunctions___spec__2(size_t, size_t, lean_object*); @@ -183,6 +182,7 @@ lean_object* l___private_Lean_CoreM_0__Lean_Core_mkFreshNameImp(lean_object*, le static lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEqEnum___closed__8; static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__1___closed__21; uint8_t l_Lean_InductiveVal_isNested(lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__3___closed__11; lean_object* l_Lean_Elab_getBetterRef(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_DecEq_mkMatch_mkAlts___spec__8___boxed(lean_object*, lean_object*, lean_object*); @@ -224,6 +224,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_DecEq_mkEnumOfNat___lambda__1___bo extern lean_object* l_Lean_instInhabitedExpr; static lean_object* l_Lean_Elab_Deriving_DecEq_mkEnumOfNatThm___closed__4; static lean_object* l_Lean_Elab_Deriving_DecEq_mkAuxFunction___lambda__1___closed__16; +LEAN_EXPORT lean_object* l_Lean_Elab_withEnableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Command_getCurrMacroScope(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEqEnum___closed__50; static lean_object* l_Lean_Elab_Deriving_DecEq_mkAuxFunction___lambda__1___closed__9; @@ -265,11 +266,11 @@ static lean_object* l_Lean_getConstInfoInduct___at_Lean_Elab_Deriving_DecEq_mkDe lean_object* lean_mk_syntax_ident(lean_object*); static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_DecEq_mkMatch_mkAlts___spec__5___closed__1; static lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEqHeader___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_enableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__6(uint8_t, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_DecEq_initFn____x40_Lean_Elab_Deriving_DecEq___hyg_4874____closed__3; static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__1___closed__10; static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__2___closed__31; static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__2___closed__5; -LEAN_EXPORT lean_object* l_Lean_Elab_enableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_DecEq_mkMatch_mkAlts___spec__5___lambda__2___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_getConstInfoCtor___at_Lean_Elab_Deriving_DecEq_mkMatch_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_DecEq_mkDecEqEnum___closed__27; @@ -299,7 +300,6 @@ static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__2 lean_object* l_Lean_Core_transform___at_Lean_Core_betaReduce___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEqCmds___closed__10; static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__1___closed__9; -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__2___closed__10; static lean_object* l_Lean_Elab_Deriving_DecEq_initFn____x40_Lean_Elab_Deriving_DecEq___hyg_4874____closed__6; static lean_object* l_Lean_Elab_Deriving_DecEq_mkAuxFunction___lambda__1___closed__11; @@ -317,6 +317,7 @@ static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__1 static lean_object* l_Lean_Elab_Deriving_DecEq_mkAuxFunction___lambda__1___closed__15; static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__2___closed__8; lean_object* l_Lean_Expr_app___override(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__2___closed__42; static lean_object* l_Lean_getConstInfoInduct___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__1___closed__2; lean_object* l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -372,6 +373,7 @@ lean_object* l_Lean_mkArrow(lean_object*, lean_object*, lean_object*, lean_objec static lean_object* l_Lean_Elab_Deriving_DecEq_initFn____x40_Lean_Elab_Deriving_DecEq___hyg_4874____closed__9; static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_DecEq_mkMatch_mkAlts___spec__6___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_DecEq_mkEnumOfNat_mkDecTree(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__2___closed__46; LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch(lean_object*, 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_Deriving_DecEq_mkMatch_mkAlts___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -395,6 +397,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_DecEq_mkEnumOfNatThm___lambda__1__ lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_SynthInstance_removeUnusedArguments_x3f___spec__2___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_DecEq_mkAuxFunction___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEqEnum___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Function_comp___rarg(lean_object*, lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); static lean_object* l_Lean_Elab_Deriving_DecEq_mkAuxFunction___lambda__1___closed__18; @@ -428,6 +431,7 @@ lean_object* lean_array_get_size(lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_DecEq_mkMatch_mkAlts___spec__6___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEqEnum___closed__40; static lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEqEnum___closed__3; +static lean_object* l_Lean_getConstInfo___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__2___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_DecEq_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*, lean_object*); lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); @@ -448,6 +452,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_DecEq_mkEnumOfNatThm(lean_object*, static lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEqEnum___closed__39; static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_DecEq_mkMatch_mkAlts___spec__5___closed__5; static lean_object* l_Lean_Elab_Deriving_DecEq_mkAuxFunction___lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_withEnableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__5(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEqEnum___closed__42; lean_object* l_String_toSubstring_x27(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEqInstance(lean_object*, lean_object*, lean_object*, lean_object*); @@ -462,6 +467,7 @@ static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__1 static lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEqCmds___closed__9; static lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEqEnum___closed__26; LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEqCmds___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_DecEq_mkEnumOfNat_mkDecTree___closed__1; static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Deriving_DecEq_mkDecEqInstanceHandler___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -10248,7 +10254,204 @@ lean_dec(x_2); return x_10; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Deriving_DecEq_mkDecEq___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_Elab_Deriving_DecEq_mkDecEq___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_5 = l_Lean_Elab_Command_getRef(x_2, x_3, x_4); +x_6 = lean_ctor_get(x_5, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_5, 1); +lean_inc(x_7); +lean_dec(x_5); +x_8 = lean_ctor_get(x_2, 4); +lean_inc(x_8); +lean_inc(x_8); +x_9 = l_Lean_Elab_getBetterRef(x_6, x_8); +lean_dec(x_6); +x_10 = l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1(x_1, x_2, x_3, x_7); +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_12 = lean_ctor_get(x_10, 0); +x_13 = lean_ctor_get(x_10, 1); +x_14 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_12, x_8, x_2, x_3, x_13); +lean_dec(x_2); +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 0) +{ +lean_object* x_16; +x_16 = lean_ctor_get(x_14, 0); +lean_ctor_set(x_10, 1, x_16); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set_tag(x_14, 1); +lean_ctor_set(x_14, 0, x_10); +return x_14; +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_14, 0); +x_18 = lean_ctor_get(x_14, 1); +lean_inc(x_18); +lean_inc(x_17); +lean_dec(x_14); +lean_ctor_set(x_10, 1, x_17); +lean_ctor_set(x_10, 0, x_9); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_10); +lean_ctor_set(x_19, 1, 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; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_20 = lean_ctor_get(x_10, 0); +x_21 = lean_ctor_get(x_10, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_10); +x_22 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_20, x_8, x_2, x_3, x_21); +lean_dec(x_2); +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +if (lean_is_exclusive(x_22)) { + lean_ctor_release(x_22, 0); + lean_ctor_release(x_22, 1); + x_25 = x_22; +} else { + lean_dec_ref(x_22); + x_25 = lean_box(0); +} +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_9); +lean_ctor_set(x_26, 1, x_23); +if (lean_is_scalar(x_25)) { + x_27 = lean_alloc_ctor(1, 2, 0); +} else { + x_27 = x_25; + lean_ctor_set_tag(x_27, 1); +} +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_24); +return x_27; +} +} +} +static lean_object* _init_l_Lean_getConstInfo___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__2___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("unknown constant '", 18, 18); +return x_1; +} +} +static lean_object* _init_l_Lean_getConstInfo___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__2___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_getConstInfo___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__2___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; uint8_t x_6; +x_5 = lean_st_ref_get(x_3, x_4); +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; +x_7 = lean_ctor_get(x_5, 0); +x_8 = lean_ctor_get(x_5, 1); +x_9 = lean_ctor_get(x_7, 0); +lean_inc(x_9); +lean_dec(x_7); +lean_inc(x_1); +x_10 = lean_environment_find(x_9, x_1); +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; +lean_free_object(x_5); +x_11 = lean_box(0); +x_12 = l_Lean_Expr_const___override(x_1, x_11); +x_13 = l_Lean_MessageData_ofExpr(x_12); +x_14 = l_Lean_getConstInfo___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__2___closed__2; +x_15 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_13); +x_16 = l_Lean_getConstInfoCtor___at_Lean_Elab_Deriving_DecEq_mkMatch_mkAlts___spec__1___closed__2; +x_17 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_17, 0, x_15); +lean_ctor_set(x_17, 1, x_16); +x_18 = l_Lean_throwError___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__3(x_17, x_2, x_3, x_8); +return x_18; +} +else +{ +lean_object* x_19; +lean_dec(x_2); +lean_dec(x_1); +x_19 = lean_ctor_get(x_10, 0); +lean_inc(x_19); +lean_dec(x_10); +lean_ctor_set(x_5, 0, x_19); +return x_5; +} +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_20 = lean_ctor_get(x_5, 0); +x_21 = lean_ctor_get(x_5, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_5); +x_22 = lean_ctor_get(x_20, 0); +lean_inc(x_22); +lean_dec(x_20); +lean_inc(x_1); +x_23 = lean_environment_find(x_22, x_1); +if (lean_obj_tag(x_23) == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_24 = lean_box(0); +x_25 = l_Lean_Expr_const___override(x_1, x_24); +x_26 = l_Lean_MessageData_ofExpr(x_25); +x_27 = l_Lean_getConstInfo___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__2___closed__2; +x_28 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_26); +x_29 = l_Lean_getConstInfoCtor___at_Lean_Elab_Deriving_DecEq_mkMatch_mkAlts___spec__1___closed__2; +x_30 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +x_31 = l_Lean_throwError___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__3(x_30, x_2, x_3, x_21); +return x_31; +} +else +{ +lean_object* x_32; lean_object* x_33; +lean_dec(x_2); +lean_dec(x_1); +x_32 = lean_ctor_get(x_23, 0); +lean_inc(x_32); +lean_dec(x_23); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_21); +return x_33; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; @@ -10359,7 +10562,7 @@ LEAN_EXPORT lean_object* l_Lean_getConstInfoInduct___at_Lean_Elab_Deriving_DecEq lean_object* x_5; lean_inc(x_2); lean_inc(x_1); -x_5 = l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9(x_1, x_2, x_3, x_4); +x_5 = l_Lean_getConstInfo___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__2(x_1, x_2, x_3, x_4); if (lean_obj_tag(x_5) == 0) { lean_object* x_6; @@ -10415,7 +10618,7 @@ x_19 = l_Lean_getConstInfoInduct___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__1 x_20 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_20, 0, x_18); lean_ctor_set(x_20, 1, x_19); -x_21 = l_Lean_throwError___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__2(x_20, x_2, x_3, x_13); +x_21 = l_Lean_throwError___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__4(x_20, x_2, x_3, x_13); return x_21; } } @@ -10445,7 +10648,7 @@ return x_25; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_enableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__4(uint8_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_enableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__6(uint8_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; @@ -10597,7 +10800,7 @@ return x_43; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_withEnableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__3(uint8_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Elab_withEnableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__5(uint8_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; @@ -10612,7 +10815,7 @@ lean_inc(x_9); lean_dec(x_7); x_10 = lean_ctor_get_uint8(x_9, sizeof(void*)*2); lean_dec(x_9); -x_11 = l_Lean_Elab_enableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__4(x_1, x_3, x_4, x_8); +x_11 = l_Lean_Elab_enableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__6(x_1, x_3, x_4, x_8); x_12 = lean_ctor_get(x_11, 1); lean_inc(x_12); lean_dec(x_11); @@ -10627,7 +10830,7 @@ 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_enableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__4(x_10, x_3, x_4, x_15); +x_16 = l_Lean_Elab_enableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__6(x_10, x_3, x_4, x_15); lean_dec(x_4); lean_dec(x_3); x_17 = !lean_is_exclusive(x_16); @@ -10659,7 +10862,7 @@ lean_inc(x_21); x_22 = lean_ctor_get(x_13, 1); lean_inc(x_22); lean_dec(x_13); -x_23 = l_Lean_Elab_enableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__4(x_10, x_3, x_4, x_22); +x_23 = l_Lean_Elab_enableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__6(x_10, x_3, x_4, x_22); lean_dec(x_4); lean_dec(x_3); x_24 = !lean_is_exclusive(x_23); @@ -10755,7 +10958,7 @@ lean_dec(x_14); lean_dec(x_12); x_17 = 0; x_18 = l_Lean_Elab_Deriving_DecEq_mkDecEq___closed__1; -x_19 = l_Lean_Elab_withEnableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__3(x_17, x_18, x_2, x_3, x_13); +x_19 = l_Lean_Elab_withEnableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__5(x_17, x_18, x_2, x_3, x_13); if (lean_obj_tag(x_19) == 0) { uint8_t x_20; @@ -10818,7 +11021,7 @@ lean_dec(x_14); lean_dec(x_12); x_33 = 0; x_34 = l_Lean_Elab_Deriving_DecEq_mkDecEq___closed__1; -x_35 = l_Lean_Elab_withEnableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__3(x_33, x_34, x_2, x_3, x_13); +x_35 = l_Lean_Elab_withEnableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__5(x_33, x_34, x_2, x_3, x_13); if (lean_obj_tag(x_35) == 0) { uint8_t x_36; @@ -10884,7 +11087,7 @@ lean_closure_set(x_52, 1, x_50); lean_closure_set(x_52, 2, x_51); lean_closure_set(x_52, 3, x_49); x_53 = 0; -x_54 = l_Lean_Elab_withEnableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__3(x_53, x_52, x_2, x_3, x_13); +x_54 = l_Lean_Elab_withEnableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__5(x_53, x_52, x_2, x_3, x_13); if (lean_obj_tag(x_54) == 0) { uint8_t x_55; @@ -11008,7 +11211,7 @@ lean_dec(x_80); lean_dec(x_78); x_83 = 0; x_84 = l_Lean_Elab_Deriving_DecEq_mkDecEq___closed__1; -x_85 = l_Lean_Elab_withEnableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__3(x_83, x_84, x_2, x_3, x_79); +x_85 = l_Lean_Elab_withEnableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__5(x_83, x_84, x_2, x_3, x_79); if (lean_obj_tag(x_85) == 0) { lean_object* x_86; lean_object* x_87; uint8_t x_88; lean_object* x_89; lean_object* x_90; @@ -11069,7 +11272,7 @@ lean_dec(x_80); lean_dec(x_78); x_96 = 0; x_97 = l_Lean_Elab_Deriving_DecEq_mkDecEq___closed__1; -x_98 = l_Lean_Elab_withEnableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__3(x_96, x_97, x_2, x_3, x_79); +x_98 = l_Lean_Elab_withEnableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__5(x_96, x_97, x_2, x_3, x_79); if (lean_obj_tag(x_98) == 0) { lean_object* x_99; lean_object* x_100; uint8_t x_101; lean_object* x_102; lean_object* x_103; @@ -11133,7 +11336,7 @@ lean_closure_set(x_112, 1, x_110); lean_closure_set(x_112, 2, x_111); lean_closure_set(x_112, 3, x_109); x_113 = 0; -x_114 = l_Lean_Elab_withEnableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__3(x_113, x_112, x_2, x_3, x_79); +x_114 = l_Lean_Elab_withEnableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__5(x_113, x_112, x_2, x_3, x_79); if (lean_obj_tag(x_114) == 0) { lean_object* x_115; lean_object* x_116; uint8_t x_117; lean_object* x_118; lean_object* x_119; @@ -11253,11 +11456,29 @@ return x_134; } } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Deriving_DecEq_mkDecEq___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_Elab_Deriving_DecEq_mkDecEq___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Lean_throwError___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__3(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at_Lean_Elab_Deriving_DecEq_mkDecEq___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_getConstInfo___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__2(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_throwError___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__2(x_1, x_2, x_3, x_4); +x_5 = l_Lean_throwError___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__4(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } @@ -11271,25 +11492,25 @@ lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_enableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_enableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__6___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_1); lean_dec(x_1); -x_6 = l_Lean_Elab_enableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__4(x_5, x_2, x_3, x_4); +x_6 = l_Lean_Elab_enableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__6(x_5, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_2); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Elab_withEnableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___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_Lean_Elab_withEnableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___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_1); lean_dec(x_1); -x_7 = l_Lean_Elab_withEnableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__3(x_6, x_2, x_3, x_4, x_5); +x_7 = l_Lean_Elab_withEnableInfoTree___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__5(x_6, x_2, x_3, x_4, x_5); return x_7; } } @@ -15168,7 +15389,7 @@ if (lean_is_exclusive(x_1)) { x_10 = lean_box(0); } lean_inc(x_2); -x_18 = l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9(x_8, x_2, x_3, x_4); +x_18 = l_Lean_getConstInfo___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__2(x_8, x_2, x_3, x_4); if (lean_obj_tag(x_18) == 0) { lean_object* x_19; @@ -15266,7 +15487,7 @@ LEAN_EXPORT lean_object* l_Lean_isEnumType___at_Lean_Elab_Deriving_DecEq_mkDecEq { lean_object* x_5; lean_inc(x_2); -x_5 = l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9(x_1, x_2, x_3, x_4); +x_5 = l_Lean_getConstInfo___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__2(x_1, x_2, x_3, x_4); if (lean_obj_tag(x_5) == 0) { lean_object* x_6; @@ -16461,6 +16682,10 @@ l_Lean_Elab_Deriving_DecEq_mkDecEqCmds___closed__10 = _init_l_Lean_Elab_Deriving lean_mark_persistent(l_Lean_Elab_Deriving_DecEq_mkDecEqCmds___closed__10); l_Lean_Elab_Deriving_DecEq_mkDecEqCmds___closed__11 = _init_l_Lean_Elab_Deriving_DecEq_mkDecEqCmds___closed__11(); lean_mark_persistent(l_Lean_Elab_Deriving_DecEq_mkDecEqCmds___closed__11); +l_Lean_getConstInfo___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__2___closed__1 = _init_l_Lean_getConstInfo___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__2___closed__1(); +lean_mark_persistent(l_Lean_getConstInfo___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__2___closed__1); +l_Lean_getConstInfo___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__2___closed__2 = _init_l_Lean_getConstInfo___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__2___closed__2(); +lean_mark_persistent(l_Lean_getConstInfo___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__2___closed__2); l_Lean_getConstInfoInduct___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__1___closed__1 = _init_l_Lean_getConstInfoInduct___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__1___closed__1(); lean_mark_persistent(l_Lean_getConstInfoInduct___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__1___closed__1); l_Lean_getConstInfoInduct___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__1___closed__2 = _init_l_Lean_getConstInfoInduct___at_Lean_Elab_Deriving_DecEq_mkDecEq___spec__1___closed__2(); diff --git a/stage0/stdlib/Lean/Elab/Deriving/FromToJson.c b/stage0/stdlib/Lean/Elab/Deriving/FromToJson.c index cbe35a926aaf..62fff02aac01 100644 --- a/stage0/stdlib/Lean/Elab/Deriving/FromToJson.c +++ b/stage0/stdlib/Lean/Elab/Deriving/FromToJson.c @@ -42,6 +42,7 @@ static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonHeader___closed__1 static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__1___closed__14; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonHeader___closed__5; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__1___closed__16; +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__4; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6656____closed__16; LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -66,6 +67,7 @@ static lean_object* l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deri lean_object* lean_array_push(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__4(lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* l_Array_qpartition___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__5; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__1___closed__5; static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__3___closed__3; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__1___closed__13; @@ -78,6 +80,7 @@ static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___lamb lean_object* l_Lean_Elab_Deriving_mkInstanceCmds(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__1___closed__7; LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; lean_object* l_Lean_Elab_Deriving_mkDiscrs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___lambda__1___closed__12; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonAuxFunction___lambda__1___closed__7; @@ -87,7 +90,6 @@ lean_object* l_Lean_Elab_Command_elabCommand(lean_object*, lean_object*, lean_ob lean_object* lean_array_fget(lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct_mkAlts___spec__3___closed__3; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForStruct___spec__1___closed__2; -static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__7; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___lambda__1___closed__12; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___closed__5; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonHeader___closed__6; @@ -103,6 +105,7 @@ static lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Elab_Deriving_FromToJson LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_mkJsonField___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForStruct___spec__1___closed__25; static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__2___closed__13; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_isInductive___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__1___closed__40; @@ -113,12 +116,12 @@ uint8_t l_Lean_Expr_isAppOf(lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__2___closed__6; static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct_mkAlts___spec__4___lambda__1___closed__2; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonHeader___closed__11; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___lambda__1___closed__5; lean_object* l_Lean_getConstInfoInduct___at_Lean_Elab_Deriving_mkContext___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_node5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForStruct___closed__4; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonHeader___closed__24; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_stringToMessageData(lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___closed__12; @@ -141,7 +144,6 @@ static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___lambda LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__8(lean_object*, lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__2___closed__12; LEAN_EXPORT lean_object* l_Lean_getConstInfoCtor___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct_mkAlts___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Deriving_FromToJson_0__Lean_Elab_Deriving_FromToJson_mkToJsonInstance___closed__1; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___closed__2; static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__2___closed__2; @@ -162,7 +164,6 @@ lean_object* l_Array_mapMUnsafe_map___at___aux__Init__NotationExtra______macroRu static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForStruct___spec__1___closed__20; static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__3___closed__8; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___closed__9; -static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13; lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonAuxFunction___lambda__1___closed__12; static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__3___closed__4; @@ -179,20 +180,26 @@ static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonMutualBlock___closed static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__2___closed__8; lean_object* l_Lean_Elab_registerDerivingHandler(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Substring_takeRightWhileAux___at_Lean_Elab_Deriving_FromToJson_mkJsonField___spec__2___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__7; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct_mkAlts___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___lambda__1___closed__11; +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__2; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__1___closed__31; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct_mkAlts___spec__4___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Deriving_mkLet(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__3___closed__13; +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14; lean_object* l_Array_zip___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct___closed__4; +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__12; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___closed__4; lean_object* l_Lean_SourceInfo_fromRef(lean_object*, uint8_t); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__9; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__2___closed__6; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___lambda__1___closed__6; lean_object* l_Lean_MessageData_ofSyntax(lean_object*); @@ -213,8 +220,6 @@ static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonHeader___closed__1 static lean_object* l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6656____closed__13; LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_CoreM_0__Lean_Core_mkFreshNameImp(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__5; -static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___lambda__1___closed__7; static lean_object* l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6656____closed__14; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___lambda__1___closed__9; @@ -253,8 +258,8 @@ static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mk static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct_mkAlts___spec__5___lambda__1___closed__4; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__5(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13; lean_object* lean_array_to_list(lean_object*); -static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonAuxFunction___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__2___closed__2; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); @@ -290,6 +295,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForStruct(l static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForStruct___spec__1___closed__16; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__2___closed__7; lean_object* l_Lean_Syntax_node2(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8; LEAN_EXPORT lean_object* l_Substring_takeRightWhileAux___at_Lean_Elab_Deriving_FromToJson_mkJsonField___spec__2(lean_object*, lean_object*, lean_object*); lean_object* lean_string_utf8_prev(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForStruct___closed__10; @@ -300,7 +306,6 @@ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Elab_Deriving_FromT static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__1___closed__20; static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct_mkAlts___spec__5___lambda__1___closed__7; static lean_object* l_Lean_getConstInfoCtor___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct_mkAlts___spec__1___closed__2; -static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForStruct___spec__1___closed__9; static lean_object* l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6656____closed__8; lean_object* lean_mk_syntax_ident(lean_object*); @@ -317,7 +322,6 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJs LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); static lean_object* l_Lean_getConstInfoCtor___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct_mkAlts___spec__1___closed__3; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofExpr(lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct_mkAlts___spec__5___lambda__1___closed__1; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonMutualBlock___closed__2; @@ -329,9 +333,9 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJs LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct_mkAlts___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___lambda__1___closed__4; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForStruct___spec__1___closed__5; -static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; static lean_object* l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6656____closed__10; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForStruct___spec__1___closed__13; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonMutualBlock(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonHeader___closed__25; lean_object* l_Lean_LocalDecl_userName(lean_object*); @@ -340,14 +344,15 @@ lean_object* l_Lean_Syntax_node4(lean_object*, lean_object*, lean_object*, lean_ LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___lambda__1___closed__14; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__1___closed__34; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__2___closed__1; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct___closed__2; static lean_object* l___private_Lean_Elab_Deriving_FromToJson_0__Lean_Elab_Deriving_FromToJson_mkToJsonInstance___closed__2; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___lambda__1___closed__13; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonAuxFunction(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; static lean_object* l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6656____closed__17; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___lambda__1___closed__20; uint8_t l_Lean_Name_hasMacroScopes(lean_object*); @@ -363,7 +368,6 @@ static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mk static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___lambda__1___closed__8; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___lambda__1___closed__3; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___lambda__1___closed__21; -static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__9; lean_object* l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__3___closed__5; @@ -374,7 +378,6 @@ uint8_t lean_nat_dec_lt(lean_object*, lean_object*); lean_object* lean_environment_main_module(lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonHeader___closed__10; LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_Deriving_FromToJson_0__Lean_Elab_Deriving_FromToJson_mkFromJsonInstance___spec__1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__1___closed__9; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForStruct___closed__18; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct___closed__3; @@ -405,7 +408,6 @@ static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct___cl lean_object* l_Lean_Syntax_node1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForStruct___closed__17; lean_object* l_Lean_mkSepArray(lean_object*, lean_object*); -static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__12; static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__3___closed__10; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__2___closed__8; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForStruct___closed__12; @@ -425,14 +427,13 @@ uint8_t l_Lean_isStructure(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___lambda__1___closed__25; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonAuxFunction___lambda__1___closed__8; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonHeader___closed__19; +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__3; static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___closed__1; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct___closed__8; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__1___closed__29; -static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__3; lean_object* l_Lean_Name_getString_x21(lean_object*); -static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonMutualBlock(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__1___closed__4; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__1___closed__19; lean_object* lean_erase_macro_scopes(lean_object*); @@ -460,7 +461,6 @@ LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJs static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___lambda__1___closed__1; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__1___closed__2; static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct_mkAlts___spec__5___lambda__1___closed__8; -static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__4; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___closed__1; size_t lean_usize_add(size_t, size_t); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___lambda__1___closed__3; @@ -476,6 +476,7 @@ static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___lamb size_t lean_array_size(lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonAuxFunction___lambda__1___closed__3; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___lambda__1___closed__18; +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__1; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__1___closed__26; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___closed__11; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__3___closed__1; @@ -486,7 +487,6 @@ LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mk static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__2___closed__3; static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct_mkAlts___spec__5___lambda__1___closed__9; lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__2___closed__5; LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_Deriving_FromToJson_0__Lean_Elab_Deriving_FromToJson_mkToJsonInstance___spec__1(lean_object*, lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__3___closed__6; @@ -508,6 +508,7 @@ static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct___cl static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___lambda__1___closed__10; uint8_t lean_nat_dec_le(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonBody(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__6; uint8_t lean_usize_dec_lt(size_t, size_t); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___lambda__1___closed__16; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__1___closed__21; @@ -541,7 +542,6 @@ static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___clos LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct_mkAlts___spec__4___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__3___closed__4; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___closed__7; -static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__1; lean_object* l_Lean_Syntax_mkNumLit(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonHeader___closed__12; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForStruct___closed__15; @@ -4590,7 +4590,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { lean_object* x_17; uint8_t x_18; @@ -4870,7 +4870,7 @@ return x_134; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { lean_object* x_17; uint8_t x_18; @@ -5696,7 +5696,7 @@ lean_object* x_191; lean_object* x_192; lean_object* x_193; uint8_t x_194; x_191 = lean_ctor_get(x_5, 0); x_192 = lean_mk_empty_array_with_capacity(x_17); lean_inc(x_10); -x_193 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___spec__2(x_1, x_2, x_4, x_191, x_4, x_17, x_18, lean_box(0), x_192, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_193 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___spec__2(x_1, x_2, x_4, x_191, x_4, x_17, x_18, lean_box(0), x_192, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_4); x_194 = !lean_is_exclusive(x_193); if (x_194 == 0) @@ -6300,7 +6300,7 @@ x_453 = lean_array_mk(x_452); x_454 = lean_array_get_size(x_453); x_455 = lean_mk_empty_array_with_capacity(x_454); lean_inc(x_10); -x_456 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___spec__3(x_1, x_2, x_450, x_453, x_453, x_454, x_18, lean_box(0), x_455, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_456 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___spec__3(x_1, x_2, x_450, x_453, x_453, x_454, x_18, lean_box(0), x_455, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_453); x_457 = !lean_is_exclusive(x_456); if (x_457 == 0) @@ -7133,11 +7133,11 @@ lean_dec(x_1); return x_15; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { lean_object* x_17; -x_17 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_17 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_15); lean_dec(x_13); lean_dec(x_12); @@ -7150,11 +7150,11 @@ lean_dec(x_1); return x_17; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { lean_object* x_17; -x_17 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_17 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_15); lean_dec(x_13); lean_dec(x_12); @@ -9664,7 +9664,7 @@ goto _start; } } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__1() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__1() { _start: { lean_object* x_1; @@ -9672,61 +9672,61 @@ x_1 = lean_mk_string_unchecked("fromJson\?", 9, 9); return x_1; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__2() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__1; +x_1 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__1; x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__3() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__1; +x_2 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__4() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Elab_Deriving_FromToJson_mkToJsonHeader___closed__1; x_2 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonHeader___closed__1; -x_3 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__1; +x_3 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__1; x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); return x_4; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__5() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__4; +x_2 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__4; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__6() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__5; +x_2 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__5; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__7() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__7() { _start: { lean_object* x_1; @@ -9734,17 +9734,17 @@ x_1 = lean_mk_string_unchecked("term__[_]_!", 11, 11); return x_1; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__7; +x_2 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__7; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__9() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__9() { _start: { lean_object* x_1; @@ -9752,26 +9752,26 @@ x_1 = lean_mk_string_unchecked("jsons", 5, 5); return x_1; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__9; +x_1 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__9; x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__9; +x_2 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__9; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__12() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__12() { _start: { lean_object* x_1; @@ -9779,17 +9779,17 @@ x_1 = lean_mk_string_unchecked("group", 5, 5); return x_1; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__12; +x_2 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__12; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14() { _start: { lean_object* x_1; @@ -9797,7 +9797,7 @@ x_1 = lean_mk_string_unchecked("!", 1, 1); return x_1; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { lean_object* x_16; uint8_t x_17; @@ -9842,29 +9842,29 @@ x_35 = lean_ctor_get(x_33, 0); lean_inc(x_35); lean_dec(x_33); x_36 = lean_environment_main_module(x_35); -x_37 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__3; +x_37 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__3; lean_inc(x_30); lean_inc(x_36); x_38 = l_Lean_addMacroScope(x_36, x_37, x_30); x_39 = lean_box(0); -x_40 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__2; -x_41 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__6; +x_40 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__2; +x_41 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__6; lean_inc(x_29); x_42 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_42, 0, x_29); lean_ctor_set(x_42, 1, x_40); lean_ctor_set(x_42, 2, x_38); lean_ctor_set(x_42, 3, x_41); -x_43 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; +x_43 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; x_44 = l_Lean_addMacroScope(x_36, x_43, x_30); -x_45 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; +x_45 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; lean_inc(x_29); x_46 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_46, 0, x_29); lean_ctor_set(x_46, 1, x_45); lean_ctor_set(x_46, 2, x_44); lean_ctor_set(x_46, 3, x_39); -x_47 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13; +x_47 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13; x_48 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonHeader___closed__25; lean_inc(x_29); x_49 = lean_alloc_ctor(1, 3, 0); @@ -9885,12 +9885,12 @@ lean_inc(x_29); lean_ctor_set_tag(x_20, 2); lean_ctor_set(x_20, 1, x_54); lean_ctor_set(x_20, 0, x_29); -x_55 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14; +x_55 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14; lean_inc(x_29); x_56 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_56, 0, x_29); lean_ctor_set(x_56, 1, x_55); -x_57 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8; +x_57 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8; lean_inc(x_49); lean_inc(x_29); x_58 = l_Lean_Syntax_node7(x_29, x_57, x_46, x_49, x_31, x_53, x_20, x_49, x_56); @@ -9924,29 +9924,29 @@ x_70 = lean_ctor_get(x_68, 0); lean_inc(x_70); lean_dec(x_68); x_71 = lean_environment_main_module(x_70); -x_72 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__3; +x_72 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__3; lean_inc(x_30); lean_inc(x_71); x_73 = l_Lean_addMacroScope(x_71, x_72, x_30); x_74 = lean_box(0); -x_75 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__2; -x_76 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__6; +x_75 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__2; +x_76 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__6; lean_inc(x_29); x_77 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_77, 0, x_29); lean_ctor_set(x_77, 1, x_75); lean_ctor_set(x_77, 2, x_73); lean_ctor_set(x_77, 3, x_76); -x_78 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; +x_78 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; x_79 = l_Lean_addMacroScope(x_71, x_78, x_30); -x_80 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; +x_80 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; lean_inc(x_29); x_81 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_81, 0, x_29); lean_ctor_set(x_81, 1, x_80); lean_ctor_set(x_81, 2, x_79); lean_ctor_set(x_81, 3, x_74); -x_82 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13; +x_82 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13; x_83 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonHeader___closed__25; lean_inc(x_29); x_84 = lean_alloc_ctor(1, 3, 0); @@ -9967,12 +9967,12 @@ lean_inc(x_29); lean_ctor_set_tag(x_20, 2); lean_ctor_set(x_20, 1, x_90); lean_ctor_set(x_20, 0, x_29); -x_91 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14; +x_91 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14; lean_inc(x_29); x_92 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_92, 0, x_29); lean_ctor_set(x_92, 1, x_91); -x_93 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8; +x_93 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8; lean_inc(x_84); lean_inc(x_29); x_94 = l_Lean_Syntax_node7(x_29, x_93, x_81, x_84, x_86, x_89, x_20, x_84, x_92); @@ -10016,17 +10016,17 @@ x_112 = lean_ctor_get(x_110, 0); lean_inc(x_112); lean_dec(x_110); x_113 = lean_environment_main_module(x_112); -x_114 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; +x_114 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; x_115 = l_Lean_addMacroScope(x_113, x_114, x_107); x_116 = lean_box(0); -x_117 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; +x_117 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; lean_inc(x_106); x_118 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_118, 0, x_106); lean_ctor_set(x_118, 1, x_117); lean_ctor_set(x_118, 2, x_115); lean_ctor_set(x_118, 3, x_116); -x_119 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13; +x_119 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13; x_120 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonHeader___closed__25; lean_inc(x_106); x_121 = lean_alloc_ctor(1, 3, 0); @@ -10047,12 +10047,12 @@ lean_inc(x_106); lean_ctor_set_tag(x_20, 2); lean_ctor_set(x_20, 1, x_126); lean_ctor_set(x_20, 0, x_106); -x_127 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14; +x_127 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14; lean_inc(x_106); x_128 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_128, 0, x_106); lean_ctor_set(x_128, 1, x_127); -x_129 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8; +x_129 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8; lean_inc(x_121); lean_inc(x_106); x_130 = l_Lean_Syntax_node7(x_106, x_129, x_118, x_121, x_108, x_125, x_20, x_121, x_128); @@ -10087,17 +10087,17 @@ x_142 = lean_ctor_get(x_140, 0); lean_inc(x_142); lean_dec(x_140); x_143 = lean_environment_main_module(x_142); -x_144 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; +x_144 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; x_145 = l_Lean_addMacroScope(x_143, x_144, x_107); x_146 = lean_box(0); -x_147 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; +x_147 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; lean_inc(x_106); x_148 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_148, 0, x_106); lean_ctor_set(x_148, 1, x_147); lean_ctor_set(x_148, 2, x_145); lean_ctor_set(x_148, 3, x_146); -x_149 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13; +x_149 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13; x_150 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonHeader___closed__25; lean_inc(x_106); x_151 = lean_alloc_ctor(1, 3, 0); @@ -10118,12 +10118,12 @@ lean_inc(x_106); lean_ctor_set_tag(x_20, 2); lean_ctor_set(x_20, 1, x_157); lean_ctor_set(x_20, 0, x_106); -x_158 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14; +x_158 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14; lean_inc(x_106); x_159 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_159, 0, x_106); lean_ctor_set(x_159, 1, x_158); -x_160 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8; +x_160 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8; lean_inc(x_151); lean_inc(x_106); x_161 = l_Lean_Syntax_node7(x_106, x_160, x_148, x_151, x_153, x_156, x_20, x_151, x_159); @@ -10185,29 +10185,29 @@ x_183 = lean_ctor_get(x_180, 0); lean_inc(x_183); lean_dec(x_180); x_184 = lean_environment_main_module(x_183); -x_185 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__3; +x_185 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__3; lean_inc(x_178); lean_inc(x_184); x_186 = l_Lean_addMacroScope(x_184, x_185, x_178); x_187 = lean_box(0); -x_188 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__2; -x_189 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__6; +x_188 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__2; +x_189 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__6; lean_inc(x_177); x_190 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_190, 0, x_177); lean_ctor_set(x_190, 1, x_188); lean_ctor_set(x_190, 2, x_186); lean_ctor_set(x_190, 3, x_189); -x_191 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; +x_191 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; x_192 = l_Lean_addMacroScope(x_184, x_191, x_178); -x_193 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; +x_193 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; lean_inc(x_177); x_194 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_194, 0, x_177); lean_ctor_set(x_194, 1, x_193); lean_ctor_set(x_194, 2, x_192); lean_ctor_set(x_194, 3, x_187); -x_195 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13; +x_195 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13; x_196 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonHeader___closed__25; lean_inc(x_177); x_197 = lean_alloc_ctor(1, 3, 0); @@ -10233,12 +10233,12 @@ lean_inc(x_177); x_204 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_204, 0, x_177); lean_ctor_set(x_204, 1, x_203); -x_205 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14; +x_205 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14; lean_inc(x_177); x_206 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_206, 0, x_177); lean_ctor_set(x_206, 1, x_205); -x_207 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8; +x_207 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8; lean_inc(x_197); lean_inc(x_177); x_208 = l_Lean_Syntax_node7(x_177, x_207, x_194, x_197, x_199, x_202, x_204, x_197, x_206); @@ -10287,17 +10287,17 @@ x_226 = lean_ctor_get(x_223, 0); lean_inc(x_226); lean_dec(x_223); x_227 = lean_environment_main_module(x_226); -x_228 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; +x_228 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; x_229 = l_Lean_addMacroScope(x_227, x_228, x_221); x_230 = lean_box(0); -x_231 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; +x_231 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; lean_inc(x_220); x_232 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_232, 0, x_220); lean_ctor_set(x_232, 1, x_231); lean_ctor_set(x_232, 2, x_229); lean_ctor_set(x_232, 3, x_230); -x_233 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13; +x_233 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13; x_234 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonHeader___closed__25; lean_inc(x_220); x_235 = lean_alloc_ctor(1, 3, 0); @@ -10323,12 +10323,12 @@ lean_inc(x_220); x_242 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_242, 0, x_220); lean_ctor_set(x_242, 1, x_241); -x_243 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14; +x_243 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14; lean_inc(x_220); x_244 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_244, 0, x_220); lean_ctor_set(x_244, 1, x_243); -x_245 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8; +x_245 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8; lean_inc(x_235); lean_inc(x_220); x_246 = l_Lean_Syntax_node7(x_220, x_245, x_232, x_235, x_237, x_240, x_242, x_235, x_244); @@ -10806,9 +10806,9 @@ lean_inc(x_17); x_69 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_69, 0, x_17); lean_ctor_set(x_69, 1, x_68); -x_70 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; +x_70 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; x_71 = l_Lean_addMacroScope(x_23, x_70, x_18); -x_72 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; +x_72 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; lean_inc(x_17); x_73 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_73, 0, x_17); @@ -11017,9 +11017,9 @@ lean_inc(x_17); x_161 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_161, 0, x_17); lean_ctor_set(x_161, 1, x_160); -x_162 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; +x_162 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; x_163 = l_Lean_addMacroScope(x_115, x_162, x_18); -x_164 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; +x_164 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; lean_inc(x_17); x_165 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_165, 0, x_17); @@ -11322,7 +11322,7 @@ lean_object* x_33; lean_object* x_34; uint8_t x_35; x_33 = lean_mk_syntax_ident(x_32); lean_inc(x_11); lean_inc(x_30); -x_34 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3(x_2, x_22, x_33, x_22, x_30, x_16, lean_box(0), x_31, x_7, x_8, x_9, x_10, x_11, x_12, x_21); +x_34 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3(x_2, x_22, x_33, x_22, x_30, x_16, lean_box(0), x_31, x_7, x_8, x_9, x_10, x_11, x_12, x_21); lean_dec(x_22); x_35 = !lean_is_exclusive(x_34); if (x_35 == 0) @@ -12113,11 +12113,11 @@ x_6 = l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyFo return x_6; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { lean_object* x_16; -x_16 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +x_16 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); lean_dec(x_14); lean_dec(x_12); lean_dec(x_11); @@ -18624,34 +18624,34 @@ l_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___closed__12 = _init_l_L lean_mark_persistent(l_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___closed__12); l_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___closed__13 = _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___closed__13(); lean_mark_persistent(l_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___closed__13); -l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__1 = _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__1(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__1); -l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__2 = _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__2(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__2); -l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__3 = _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__3(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__3); -l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__4 = _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__4(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__4); -l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__5 = _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__5(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__5); -l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__6 = _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__6(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__6); -l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__7 = _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__7(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__7); -l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8 = _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8); -l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__9 = _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__9(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__9); -l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10 = _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10); -l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11 = _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11); -l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__12 = _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__12(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__12); -l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13 = _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13); -l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14 = _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14); +l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__1 = _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__1(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__1); +l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__2 = _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__2(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__2); +l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__3 = _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__3(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__3); +l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__4 = _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__4(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__4); +l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__5 = _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__5(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__5); +l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__6 = _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__6(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__6); +l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__7 = _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__7(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__7); +l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8 = _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8); +l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__9 = _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__9(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__9); +l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10 = _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10); +l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11 = _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11); +l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__12 = _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__12(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__12); +l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13 = _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13); +l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14 = _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14); l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__2___closed__1 = _init_l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__2___closed__1(); lean_mark_persistent(l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__2___closed__1); l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__2___closed__2 = _init_l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__2___closed__2(); diff --git a/stage0/stdlib/Lean/Elab/Deriving/Inhabited.c b/stage0/stdlib/Lean/Elab/Deriving/Inhabited.c index 5022037f9450..d8137370c783 100644 --- a/stage0/stdlib/Lean/Elab/Deriving/Inhabited.c +++ b/stage0/stdlib/Lean/Elab/Deriving/Inhabited.c @@ -14,6 +14,7 @@ extern "C" { #endif LEAN_EXPORT lean_object* l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_collectUsedLocalsInsts___spec__5___rarg___lambda__1(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmdWith___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); @@ -21,10 +22,10 @@ static lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Elab_Deriving static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Deriving_Inhabited___hyg_2632____closed__3; LEAN_EXPORT lean_object* l_Lean_RBNode_ins___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_collectUsedLocalsInsts___spec__3(lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmd_x3f___spec__1___closed__1; -static lean_object* l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__3___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmd_x3f___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*); static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmdWith___spec__8___closed__4; static lean_object* l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmdWith___closed__40; +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmdWith___closed__24; LEAN_EXPORT lean_object* l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_implicitBinderF; static lean_object* l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmdWith___closed__7; @@ -37,7 +38,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_m LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmd_x3f___spec__7___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_Std_Range_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmdWith___spec__7___closed__3; static lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmd_x3f___spec__1___closed__4; -LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_throwError___at___private_Lean_Elab_Command_0__Lean_Elab_Command_elabCommandUsing___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmdWith___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getConstInfoInduct___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmdWith___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -80,20 +80,25 @@ static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Deriving_Inhabited___hyg lean_object* l_Lean_Expr_fvarId_x21(lean_object*); lean_object* lean_environment_find(lean_object*, lean_object*); lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__1___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__5___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmd_x3f___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__6(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_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmdWith___spec__7___closed__1; LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmd_x3f___spec__1___lambda__1(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_addLocalInstancesForParamsAux___rarg___closed__1; LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmdWith___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_stringToMessageData(lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmd_x3f___lambda__3___closed__3; static lean_object* l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmdWith___closed__3; static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Deriving_Inhabited___hyg_2632____closed__1; static lean_object* l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmdWith___closed__22; +static lean_object* l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__5___closed__2; static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Deriving_Inhabited___hyg_2632____closed__14; LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmd_x3f___spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmdWith___closed__28; static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Deriving_Inhabited___hyg_2632____closed__4; +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_mkInhabitedInstanceHandler___boxed(lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_ptr_addr(lean_object*); lean_object* l_Lean_Meta_isTypeCorrect(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -110,7 +115,7 @@ lean_object* l_runST___rarg(lean_object*); static lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmd_x3f___spec__1___lambda__2___closed__6; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmdWith___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_registerDerivingHandler(lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_take(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmd_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_ForEachExpr_visit___spec__3(lean_object*); @@ -166,7 +171,6 @@ static lean_object* l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInha LEAN_EXPORT lean_object* l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_collectUsedLocalsInsts___spec__5___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getConstInfoInduct___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmdWith___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Deriving_Inhabited___hyg_2632____closed__12; -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_getConstInfoCtor___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmdWith___spec__3___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmd_x3f___spec__7(lean_object*); uint64_t l_Lean_Expr_hash(lean_object*); @@ -181,7 +185,6 @@ LEAN_EXPORT lean_object* l_Lean_ForEachExprWhere_visit___at___private_Lean_Elab_ static lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmd_x3f___spec__1___lambda__2___closed__7; LEAN_EXPORT lean_object* l_Lean_ForEachExprWhere_checked___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_collectUsedLocalsInsts___spec__7___rarg(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_node2(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmdWith___spec__6___closed__20; lean_object* l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmd_x3f___spec__4(lean_object*, lean_object*, lean_object*); @@ -219,12 +222,12 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_m static lean_object* l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmdWith___closed__19; static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Deriving_Inhabited___hyg_2632____closed__8; static lean_object* l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_addLocalInstancesForParamsAux___rarg___closed__3; +LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getConstInfoInduct___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmdWith___closed__36; static lean_object* l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmdWith___closed__35; lean_object* l_Lean_Expr_isFVar___boxed(lean_object*); static lean_object* l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmdWith___closed__32; -LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmd_x3f___spec__1___lambda__2___closed__1; static lean_object* l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmdWith___closed__14; lean_object* l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -289,12 +292,14 @@ uint8_t l_Lean_Name_quickCmp(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance(lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Deriving_Inhabited___hyg_2632____closed__6; +static lean_object* l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__2___closed__1; static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmdWith___spec__6___closed__11; lean_object* lean_array_uget(lean_object*, size_t); LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmd_x3f___spec__1___boxed(lean_object**); size_t lean_array_size(lean_object*); static lean_object* l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmdWith___closed__25; LEAN_EXPORT lean_object* l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_addLocalInstancesForParams___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_getConstInfo___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__2___closed__2; lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmdWith___spec__6___closed__19; lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); @@ -332,10 +337,10 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_m static lean_object* l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmdWith___closed__8; LEAN_EXPORT lean_object* l_Lean_RBTree_toList___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmd_x3f___spec__2(lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallTelescopeReducingImp___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Deriving_Inhabited___hyg_2632_(lean_object*); size_t lean_usize_land(size_t, size_t); static lean_object* l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___closed__3; -static lean_object* l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__3___closed__2; static lean_object* l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmdWith___closed__16; LEAN_EXPORT lean_object* l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_collectUsedLocalsInsts___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ForEachExprWhere_checked___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_collectUsedLocalsInsts___spec__7(lean_object*); @@ -11895,7 +11900,204 @@ x_8 = l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceU return x_8; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___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___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_5 = l_Lean_Elab_Command_getRef(x_2, x_3, x_4); +x_6 = lean_ctor_get(x_5, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_5, 1); +lean_inc(x_7); +lean_dec(x_5); +x_8 = lean_ctor_get(x_2, 4); +lean_inc(x_8); +lean_inc(x_8); +x_9 = l_Lean_Elab_getBetterRef(x_6, x_8); +lean_dec(x_6); +x_10 = l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1(x_1, x_2, x_3, x_7); +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_12 = lean_ctor_get(x_10, 0); +x_13 = lean_ctor_get(x_10, 1); +x_14 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_12, x_8, x_2, x_3, x_13); +lean_dec(x_2); +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 0) +{ +lean_object* x_16; +x_16 = lean_ctor_get(x_14, 0); +lean_ctor_set(x_10, 1, x_16); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set_tag(x_14, 1); +lean_ctor_set(x_14, 0, x_10); +return x_14; +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_14, 0); +x_18 = lean_ctor_get(x_14, 1); +lean_inc(x_18); +lean_inc(x_17); +lean_dec(x_14); +lean_ctor_set(x_10, 1, x_17); +lean_ctor_set(x_10, 0, x_9); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_10); +lean_ctor_set(x_19, 1, 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; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_20 = lean_ctor_get(x_10, 0); +x_21 = lean_ctor_get(x_10, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_10); +x_22 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_20, x_8, x_2, x_3, x_21); +lean_dec(x_2); +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +if (lean_is_exclusive(x_22)) { + lean_ctor_release(x_22, 0); + lean_ctor_release(x_22, 1); + x_25 = x_22; +} else { + lean_dec_ref(x_22); + x_25 = lean_box(0); +} +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_9); +lean_ctor_set(x_26, 1, x_23); +if (lean_is_scalar(x_25)) { + x_27 = lean_alloc_ctor(1, 2, 0); +} else { + x_27 = x_25; + lean_ctor_set_tag(x_27, 1); +} +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_24); +return x_27; +} +} +} +static lean_object* _init_l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__2___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("unknown constant '", 18, 18); +return x_1; +} +} +static lean_object* _init_l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__2___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__2___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; uint8_t x_6; +x_5 = lean_st_ref_get(x_3, x_4); +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; +x_7 = lean_ctor_get(x_5, 0); +x_8 = lean_ctor_get(x_5, 1); +x_9 = lean_ctor_get(x_7, 0); +lean_inc(x_9); +lean_dec(x_7); +lean_inc(x_1); +x_10 = lean_environment_find(x_9, x_1); +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; +lean_free_object(x_5); +x_11 = lean_box(0); +x_12 = l_Lean_Expr_const___override(x_1, x_11); +x_13 = l_Lean_MessageData_ofExpr(x_12); +x_14 = l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__2___closed__2; +x_15 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_13); +x_16 = l_Lean_getConstInfoInduct___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmdWith___spec__1___closed__2; +x_17 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_17, 0, x_15); +lean_ctor_set(x_17, 1, x_16); +x_18 = l_Lean_throwError___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__3(x_17, x_2, x_3, x_8); +return x_18; +} +else +{ +lean_object* x_19; +lean_dec(x_2); +lean_dec(x_1); +x_19 = lean_ctor_get(x_10, 0); +lean_inc(x_19); +lean_dec(x_10); +lean_ctor_set(x_5, 0, x_19); +return x_5; +} +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_20 = lean_ctor_get(x_5, 0); +x_21 = lean_ctor_get(x_5, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_5); +x_22 = lean_ctor_get(x_20, 0); +lean_inc(x_22); +lean_dec(x_20); +lean_inc(x_1); +x_23 = lean_environment_find(x_22, x_1); +if (lean_obj_tag(x_23) == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_24 = lean_box(0); +x_25 = l_Lean_Expr_const___override(x_1, x_24); +x_26 = l_Lean_MessageData_ofExpr(x_25); +x_27 = l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__2___closed__2; +x_28 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_26); +x_29 = l_Lean_getConstInfoInduct___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmdWith___spec__1___closed__2; +x_30 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +x_31 = l_Lean_throwError___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__3(x_30, x_2, x_3, x_21); +return x_31; +} +else +{ +lean_object* x_32; lean_object* x_33; +lean_dec(x_2); +lean_dec(x_1); +x_32 = lean_ctor_get(x_23, 0); +lean_inc(x_32); +lean_dec(x_23); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_21); +return x_33; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; @@ -11989,7 +12191,7 @@ LEAN_EXPORT lean_object* l_Lean_getConstInfoInduct___at___private_Lean_Elab_Deri lean_object* x_5; lean_inc(x_2); lean_inc(x_1); -x_5 = l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9(x_1, x_2, x_3, x_4); +x_5 = l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__2(x_1, x_2, x_3, x_4); if (lean_obj_tag(x_5) == 0) { lean_object* x_6; @@ -12045,7 +12247,7 @@ x_19 = l_Lean_getConstInfoInduct___at___private_Lean_Elab_Deriving_Inhabited_0__ x_20 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_20, 0, x_18); lean_ctor_set(x_20, 1, x_19); -x_21 = l_Lean_throwError___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__2(x_20, x_2, x_3, x_13); +x_21 = l_Lean_throwError___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__4(x_20, x_2, x_3, x_13); return x_21; } } @@ -12075,7 +12277,7 @@ return x_25; } } } -static lean_object* _init_l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__3___closed__1() { +static lean_object* _init_l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__5___closed__1() { _start: { uint8_t x_1; lean_object* x_2; lean_object* x_3; @@ -12086,11 +12288,11 @@ lean_ctor_set(x_3, 0, x_2); return x_3; } } -static lean_object* _init_l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__3___closed__2() { +static lean_object* _init_l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__5___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_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__3___closed__1; +x_1 = l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__5___closed__1; x_2 = lean_box(0); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -12098,7 +12300,7 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___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_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___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) { _start: { if (lean_obj_tag(x_3) == 0) @@ -12165,7 +12367,7 @@ if (x_17 == 0) lean_object* x_18; lean_object* x_19; x_18 = lean_ctor_get(x_12, 0); lean_dec(x_18); -x_19 = l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__3___closed__2; +x_19 = l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__5___closed__2; lean_ctor_set(x_12, 0, x_19); return x_12; } @@ -12175,7 +12377,7 @@ lean_object* x_20; lean_object* x_21; lean_object* x_22; x_20 = lean_ctor_get(x_12, 1); lean_inc(x_20); lean_dec(x_12); -x_21 = l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__3___closed__2; +x_21 = l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__5___closed__2; x_22 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_22, 0, x_21); lean_ctor_set(x_22, 1, x_20); @@ -12213,7 +12415,7 @@ return x_26; } } } -LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___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_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___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) { _start: { if (lean_obj_tag(x_3) == 0) @@ -12280,7 +12482,7 @@ if (x_17 == 0) lean_object* x_18; lean_object* x_19; x_18 = lean_ctor_get(x_12, 0); lean_dec(x_18); -x_19 = l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__3___closed__2; +x_19 = l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__5___closed__2; lean_ctor_set(x_12, 0, x_19); return x_12; } @@ -12290,7 +12492,7 @@ lean_object* x_20; lean_object* x_21; lean_object* x_22; x_20 = lean_ctor_get(x_12, 1); lean_inc(x_20); lean_dec(x_12); -x_21 = l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__3___closed__2; +x_21 = l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__5___closed__2; x_22 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_22, 0, x_21); lean_ctor_set(x_22, 1, x_20); @@ -12407,7 +12609,7 @@ lean_inc(x_3); lean_inc(x_2); lean_inc(x_9); lean_inc(x_1); -x_47 = l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__4(x_1, x_46, x_9, x_46, x_2, x_3, x_7); +x_47 = l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__6(x_1, x_46, x_9, x_46, x_2, x_3, x_7); if (lean_obj_tag(x_47) == 0) { lean_object* x_48; lean_object* x_49; @@ -12557,7 +12759,7 @@ x_23 = l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_24 = l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__3(x_1, x_23, x_9, x_23, x_2, x_3, x_22); +x_24 = l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__5(x_1, x_23, x_9, x_23, x_2, x_3, x_22); if (lean_obj_tag(x_24) == 0) { lean_object* x_25; lean_object* x_26; @@ -12697,11 +12899,29 @@ return x_71; } } } -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___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___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Lean_throwError___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__3(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___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_getConstInfo___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__2(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_throwError___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__2(x_1, x_2, x_3, x_4); +x_5 = l_Lean_throwError___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__4(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } @@ -13581,10 +13801,14 @@ l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_m lean_mark_persistent(l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmd_x3f___lambda__3___closed__4); l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmd_x3f___lambda__3___closed__5 = _init_l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmd_x3f___lambda__3___closed__5(); lean_mark_persistent(l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmd_x3f___lambda__3___closed__5); -l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__3___closed__1 = _init_l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__3___closed__1(); -lean_mark_persistent(l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__3___closed__1); -l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__3___closed__2 = _init_l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__3___closed__2(); -lean_mark_persistent(l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__3___closed__2); +l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__2___closed__1 = _init_l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__2___closed__1(); +lean_mark_persistent(l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__2___closed__1); +l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__2___closed__2 = _init_l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__2___closed__2(); +lean_mark_persistent(l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__2___closed__2); +l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__5___closed__1 = _init_l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__5___closed__1(); +lean_mark_persistent(l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__5___closed__1); +l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__5___closed__2 = _init_l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__5___closed__2(); +lean_mark_persistent(l_List_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___spec__5___closed__2); l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___closed__1 = _init_l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___closed__1(); lean_mark_persistent(l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___closed__1); l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___closed__2 = _init_l___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstance___closed__2(); diff --git a/stage0/stdlib/Lean/Elab/Deriving/TypeName.c b/stage0/stdlib/Lean/Elab/Deriving/TypeName.c index 7d0702721839..21979efcc20a 100644 --- a/stage0/stdlib/Lean/Elab/Deriving/TypeName.c +++ b/stage0/stdlib/Lean/Elab/Deriving/TypeName.c @@ -14,136 +14,362 @@ extern "C" { #endif lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__64; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__17; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__52; lean_object* l_Lean_Syntax_mkNameLit(lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__52; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__78; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__22; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__58; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__27; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___closed__2; lean_object* lean_mk_empty_array_with_capacity(lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__20; LEAN_EXPORT lean_object* l___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__74; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__42; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__72; +static lean_object* l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_ConstantInfo_levelParams(lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__73; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__48; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__33; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__3; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___closed__4; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__67; lean_object* l_Lean_Elab_Command_getMainModule___rarg(lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__70; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__71; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__8; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__41; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__65; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__26; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__24; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__40; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__65; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__62; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__73; lean_object* l_Lean_Elab_Command_elabCommand(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__61; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__39; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__5; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__35; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__50; +lean_object* lean_environment_find(lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__57; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__7; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__35; lean_object* l_Lean_Syntax_node5(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_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__10; +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__45; lean_object* l_Lean_stringToMessageData(lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__59; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__14; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__46; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__60; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__74; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__68; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__79; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__11; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__10; LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Deriving_TypeName___hyg_685_(lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__34; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__60; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__31; lean_object* l_Lean_Elab_registerDerivingHandler(lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__21; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__27; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__2; lean_object* l_Lean_SourceInfo_fromRef(lean_object*, uint8_t); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__63; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__20; lean_object* l_Lean_Syntax_node6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__44; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__4; lean_object* l_Lean_Elab_Command_getRef(lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__1; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__36; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__57; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__66; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__6; lean_object* l_Lean_mkCIdentFrom(lean_object*, lean_object*, uint8_t); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Elab_getBetterRef(lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__46; lean_object* l_Lean_quoteNameMk(lean_object*); +lean_object* lean_st_ref_get(lean_object*, lean_object*); uint8_t l_List_isEmpty___rarg(lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__17; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__2___closed__1; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__72; lean_object* l_Lean_Syntax_node3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__32; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__5; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__39; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__2___closed__1; +static lean_object* l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__4; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__77; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__15; lean_object* l_Lean_Elab_Command_getCurrMacroScope(lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__31; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__12; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__25; lean_object* l_Lean_addMacroScope(lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__54; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__25; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__23; +static lean_object* l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__3; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); lean_object* l_Lean_Syntax_node2(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__2; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__1; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__37; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__75; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__44; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__45; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__30; -lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(lean_object*, 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_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__32; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__16; +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__61; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__76; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__26; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofExpr(lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__33; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__59; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__64; lean_object* l_Lean_Syntax_node4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__58; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__47; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__12; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__70; lean_object* l_Lean_Elab_Command_withFreshMacroScope___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__43; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__53; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__3; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__18; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__28; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__38; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__14; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__54; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__78; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Init_Meta_0__Lean_getEscapedNameParts_x3f(lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__13; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__7; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__51; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__76; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__16; +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__28; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__22; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__9; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__21; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__34; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__41; lean_object* l_Lean_Syntax_node1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__79; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___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_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__24; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__67; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__77; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__38; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__4; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__43; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__30; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___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_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__23; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__53; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__37; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__50; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__42; +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__63; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__51; lean_object* l_String_intercalate(lean_object*, lean_object*); lean_object* lean_array_mk(lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__29; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__75; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__13; size_t lean_usize_add(size_t, size_t); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__55; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__56; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__40; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__66; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__2; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__19; lean_object* lean_array_uget(lean_object*, size_t); size_t lean_array_size(lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__19; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__6; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__29; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__8; lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__47; +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_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__49; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__56; lean_object* lean_string_append(lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__68; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__62; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__9; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__55; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___closed__3; uint8_t lean_usize_dec_lt(size_t, size_t); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__49; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__69; +static lean_object* l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__1; +lean_object* l_Lean_throwError___at_Lean_withSetOptionIn___spec__7(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__18; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__71; lean_object* l_String_toSubstring_x27(lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__15; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__3; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__11; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__48; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___closed__1; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__36; static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Deriving_TypeName___hyg_685____closed__1; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__4; -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__1() { +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__69; +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___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; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_5 = l_Lean_Elab_Command_getRef(x_2, x_3, x_4); +x_6 = lean_ctor_get(x_5, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_5, 1); +lean_inc(x_7); +lean_dec(x_5); +x_8 = lean_ctor_get(x_2, 4); +lean_inc(x_8); +lean_inc(x_8); +x_9 = l_Lean_Elab_getBetterRef(x_6, x_8); +lean_dec(x_6); +x_10 = l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1(x_1, x_2, x_3, x_7); +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_12 = lean_ctor_get(x_10, 0); +x_13 = lean_ctor_get(x_10, 1); +x_14 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_12, x_8, x_2, x_3, x_13); +lean_dec(x_2); +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 0) +{ +lean_object* x_16; +x_16 = lean_ctor_get(x_14, 0); +lean_ctor_set(x_10, 1, x_16); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set_tag(x_14, 1); +lean_ctor_set(x_14, 0, x_10); +return x_14; +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_14, 0); +x_18 = lean_ctor_get(x_14, 1); +lean_inc(x_18); +lean_inc(x_17); +lean_dec(x_14); +lean_ctor_set(x_10, 1, x_17); +lean_ctor_set(x_10, 0, x_9); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_10); +lean_ctor_set(x_19, 1, 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; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_20 = lean_ctor_get(x_10, 0); +x_21 = lean_ctor_get(x_10, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_10); +x_22 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_20, x_8, x_2, x_3, x_21); +lean_dec(x_2); +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +if (lean_is_exclusive(x_22)) { + lean_ctor_release(x_22, 0); + lean_ctor_release(x_22, 1); + x_25 = x_22; +} else { + lean_dec_ref(x_22); + x_25 = lean_box(0); +} +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_9); +lean_ctor_set(x_26, 1, x_23); +if (lean_is_scalar(x_25)) { + x_27 = lean_alloc_ctor(1, 2, 0); +} else { + x_27 = x_25; + lean_ctor_set_tag(x_27, 1); +} +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_24); +return x_27; +} +} +} +static lean_object* _init_l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("unknown constant '", 18, 18); +return x_1; +} +} +static lean_object* _init_l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("'", 1, 1); +return x_1; +} +} +static lean_object* _init_l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__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_3, x_4); +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; +x_7 = lean_ctor_get(x_5, 0); +x_8 = lean_ctor_get(x_5, 1); +x_9 = lean_ctor_get(x_7, 0); +lean_inc(x_9); +lean_dec(x_7); +lean_inc(x_1); +x_10 = lean_environment_find(x_9, x_1); +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; +lean_free_object(x_5); +x_11 = lean_box(0); +x_12 = l_Lean_Expr_const___override(x_1, x_11); +x_13 = l_Lean_MessageData_ofExpr(x_12); +x_14 = l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__2; +x_15 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_13); +x_16 = l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__4; +x_17 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_17, 0, x_15); +lean_ctor_set(x_17, 1, x_16); +x_18 = l_Lean_throwError___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__2(x_17, x_2, x_3, x_8); +return x_18; +} +else +{ +lean_object* x_19; +lean_dec(x_2); +lean_dec(x_1); +x_19 = lean_ctor_get(x_10, 0); +lean_inc(x_19); +lean_dec(x_10); +lean_ctor_set(x_5, 0, x_19); +return x_5; +} +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_20 = lean_ctor_get(x_5, 0); +x_21 = lean_ctor_get(x_5, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_5); +x_22 = lean_ctor_get(x_20, 0); +lean_inc(x_22); +lean_dec(x_20); +lean_inc(x_1); +x_23 = lean_environment_find(x_22, x_1); +if (lean_obj_tag(x_23) == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_24 = lean_box(0); +x_25 = l_Lean_Expr_const___override(x_1, x_24); +x_26 = l_Lean_MessageData_ofExpr(x_25); +x_27 = l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__2; +x_28 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_26); +x_29 = l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__4; +x_30 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +x_31 = l_Lean_throwError___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__2(x_30, x_2, x_3, x_21); +return x_31; +} +else +{ +lean_object* x_32; lean_object* x_33; +lean_dec(x_2); +lean_dec(x_1); +x_32 = lean_ctor_get(x_23, 0); +lean_inc(x_32); +lean_dec(x_23); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_21); +return x_33; +} +} +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__1() { _start: { lean_object* x_1; @@ -151,17 +377,17 @@ x_1 = lean_mk_string_unchecked("null", 4, 4); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__2() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___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_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__1; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___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_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__3() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__3() { _start: { lean_object* x_1; @@ -169,7 +395,7 @@ x_1 = lean_mk_string_unchecked("Lean", 4, 4); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__4() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__4() { _start: { lean_object* x_1; @@ -177,7 +403,7 @@ x_1 = lean_mk_string_unchecked("Parser", 6, 6); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__5() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__5() { _start: { lean_object* x_1; @@ -185,7 +411,7 @@ x_1 = lean_mk_string_unchecked("Command", 7, 7); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__6() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__6() { _start: { lean_object* x_1; @@ -193,19 +419,19 @@ x_1 = lean_mk_string_unchecked("declaration", 11, 11); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__7() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__3; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__4; -x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__5; -x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__6; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__3; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__4; +x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__5; +x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__6; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__8() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__8() { _start: { lean_object* x_1; @@ -213,19 +439,19 @@ x_1 = lean_mk_string_unchecked("declModifiers", 13, 13); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__9() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__3; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__4; -x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__5; -x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__8; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__3; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__4; +x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__5; +x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__8; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__10() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__10() { _start: { lean_object* x_1; lean_object* x_2; @@ -234,7 +460,7 @@ x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__11() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__11() { _start: { lean_object* x_1; @@ -242,19 +468,19 @@ x_1 = lean_mk_string_unchecked("unsafe", 6, 6); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__12() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__3; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__4; -x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__5; -x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__11; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__3; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__4; +x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__5; +x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__11; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__13() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__13() { _start: { lean_object* x_1; @@ -262,19 +488,19 @@ x_1 = lean_mk_string_unchecked("definition", 10, 10); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__14() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__3; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__4; -x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__5; -x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__13; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__3; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__4; +x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__5; +x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__13; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__15() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__15() { _start: { lean_object* x_1; @@ -282,7 +508,7 @@ x_1 = lean_mk_string_unchecked("def", 3, 3); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__16() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__16() { _start: { lean_object* x_1; @@ -290,19 +516,19 @@ x_1 = lean_mk_string_unchecked("declId", 6, 6); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__17() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__17() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__3; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__4; -x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__5; -x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__16; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__3; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__4; +x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__5; +x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__16; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__18() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__18() { _start: { lean_object* x_1; @@ -310,26 +536,26 @@ x_1 = lean_mk_string_unchecked("instImpl", 8, 8); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__19() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__19() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__18; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__18; x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__20() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__20() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__18; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__18; 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_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__21() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__21() { _start: { lean_object* x_1; @@ -337,19 +563,19 @@ x_1 = lean_mk_string_unchecked("optDeclSig", 10, 10); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__22() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__22() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__3; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__4; -x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__5; -x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__21; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__3; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__4; +x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__5; +x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__21; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__23() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__23() { _start: { lean_object* x_1; @@ -357,7 +583,7 @@ x_1 = lean_mk_string_unchecked("Term", 4, 4); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__24() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__24() { _start: { lean_object* x_1; @@ -365,19 +591,19 @@ x_1 = lean_mk_string_unchecked("typeSpec", 8, 8); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__25() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__25() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__3; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__4; -x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__23; -x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__24; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__3; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__4; +x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__23; +x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__24; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__26() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__26() { _start: { lean_object* x_1; @@ -385,7 +611,7 @@ x_1 = lean_mk_string_unchecked(":", 1, 1); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__27() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__27() { _start: { lean_object* x_1; @@ -393,19 +619,19 @@ x_1 = lean_mk_string_unchecked("app", 3, 3); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__28() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__28() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__3; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__4; -x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__23; -x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__27; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__3; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__4; +x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__23; +x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__27; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__29() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__29() { _start: { lean_object* x_1; @@ -413,72 +639,72 @@ x_1 = lean_mk_string_unchecked("TypeName", 8, 8); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__30() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__30() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__29; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__29; x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__31() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__31() { _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_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__29; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__29; 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_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__32() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__32() { _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_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__31; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__31; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__33() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__33() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__31; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__31; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__34() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___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_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__33; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__33; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__35() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__35() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__32; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__34; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__32; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__34; 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_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__36() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__36() { _start: { lean_object* x_1; @@ -486,19 +712,19 @@ x_1 = lean_mk_string_unchecked("explicit", 8, 8); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__37() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__37() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__3; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__4; -x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__23; -x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__36; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__3; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__4; +x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__23; +x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__36; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__38() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__38() { _start: { lean_object* x_1; @@ -506,7 +732,7 @@ x_1 = lean_mk_string_unchecked("@", 1, 1); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__39() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__39() { _start: { lean_object* x_1; @@ -514,19 +740,19 @@ x_1 = lean_mk_string_unchecked("declValSimple", 13, 13); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__40() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__40() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__3; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__4; -x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__5; -x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__39; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__3; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__4; +x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__5; +x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__39; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__41() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__41() { _start: { lean_object* x_1; @@ -534,7 +760,7 @@ x_1 = lean_mk_string_unchecked(":=", 2, 2); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__42() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__42() { _start: { lean_object* x_1; @@ -542,19 +768,19 @@ x_1 = lean_mk_string_unchecked("dotIdent", 8, 8); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__43() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__43() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__3; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__4; -x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__23; -x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__42; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__3; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__4; +x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__23; +x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__42; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__44() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__44() { _start: { lean_object* x_1; @@ -562,7 +788,7 @@ x_1 = lean_mk_string_unchecked(".", 1, 1); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__45() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__45() { _start: { lean_object* x_1; @@ -570,26 +796,26 @@ x_1 = lean_mk_string_unchecked("mk", 2, 2); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__46() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__46() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__45; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__45; x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__47() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__47() { _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_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__45; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__45; 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_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__48() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__48() { _start: { lean_object* x_1; @@ -597,19 +823,19 @@ x_1 = lean_mk_string_unchecked("hole", 4, 4); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__49() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__49() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__3; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__4; -x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__23; -x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__48; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__3; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__4; +x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__23; +x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__48; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__50() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__50() { _start: { lean_object* x_1; @@ -617,7 +843,7 @@ x_1 = lean_mk_string_unchecked("_", 1, 1); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__51() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__51() { _start: { lean_object* x_1; @@ -625,7 +851,7 @@ x_1 = lean_mk_string_unchecked("Termination", 11, 11); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__52() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__52() { _start: { lean_object* x_1; @@ -633,19 +859,19 @@ x_1 = lean_mk_string_unchecked("suffix", 6, 6); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__53() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__53() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__3; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__4; -x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__51; -x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__52; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__3; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__4; +x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__51; +x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__52; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__54() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__54() { _start: { lean_object* x_1; @@ -653,19 +879,19 @@ x_1 = lean_mk_string_unchecked("attributes", 10, 10); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__55() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__55() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__3; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__4; -x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__23; -x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__54; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__3; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__4; +x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__23; +x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__54; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__56() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__56() { _start: { lean_object* x_1; @@ -673,7 +899,7 @@ x_1 = lean_mk_string_unchecked("@[", 2, 2); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__57() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__57() { _start: { lean_object* x_1; @@ -681,19 +907,19 @@ x_1 = lean_mk_string_unchecked("attrInstance", 12, 12); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__58() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__58() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__3; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__4; -x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__23; -x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__57; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__3; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__4; +x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__23; +x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__57; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__59() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__59() { _start: { lean_object* x_1; @@ -701,19 +927,19 @@ x_1 = lean_mk_string_unchecked("attrKind", 8, 8); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__60() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__60() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__3; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__4; -x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__23; -x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__59; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__3; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__4; +x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__23; +x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__59; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__61() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__61() { _start: { lean_object* x_1; @@ -721,7 +947,7 @@ x_1 = lean_mk_string_unchecked("Attr", 4, 4); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__62() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__62() { _start: { lean_object* x_1; @@ -729,19 +955,19 @@ x_1 = lean_mk_string_unchecked("simple", 6, 6); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__63() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__63() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__3; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__4; -x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__61; -x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__62; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__3; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__4; +x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__61; +x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__62; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__64() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__64() { _start: { lean_object* x_1; @@ -749,26 +975,26 @@ x_1 = lean_mk_string_unchecked("implemented_by", 14, 14); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__65() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__65() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__64; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__64; x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__66() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__66() { _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_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__64; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__64; 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_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__67() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__67() { _start: { lean_object* x_1; @@ -776,7 +1002,7 @@ x_1 = lean_mk_string_unchecked("]", 1, 1); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__68() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__68() { _start: { lean_object* x_1; @@ -784,19 +1010,19 @@ x_1 = lean_mk_string_unchecked("opaque", 6, 6); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__69() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__69() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__3; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__4; -x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__5; -x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__68; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__3; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__4; +x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__5; +x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__68; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__70() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__70() { _start: { lean_object* x_1; @@ -804,26 +1030,26 @@ x_1 = lean_mk_string_unchecked("inst", 4, 4); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__71() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__71() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__70; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__70; x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__72() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__72() { _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_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__70; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__70; 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_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__73() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__73() { _start: { lean_object* x_1; @@ -831,19 +1057,19 @@ x_1 = lean_mk_string_unchecked("declSig", 7, 7); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__74() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__74() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__3; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__4; -x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__5; -x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__73; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__3; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__4; +x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__5; +x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__73; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__75() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__75() { _start: { lean_object* x_1; @@ -851,19 +1077,19 @@ x_1 = lean_mk_string_unchecked("instance", 8, 8); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__76() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__76() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__3; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__4; -x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__5; -x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__75; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__3; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__4; +x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__5; +x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__75; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__77() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__77() { _start: { lean_object* x_1; @@ -871,19 +1097,19 @@ x_1 = lean_mk_string_unchecked("quotedName", 10, 10); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__78() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__78() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__3; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__4; -x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__23; -x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__77; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__3; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__4; +x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__23; +x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__77; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__79() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__79() { _start: { lean_object* x_1; @@ -891,7 +1117,7 @@ x_1 = lean_mk_string_unchecked("`", 1, 1); return x_1; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___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_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___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; @@ -918,67 +1144,67 @@ if (x_16 == 0) { lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; 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; x_17 = lean_ctor_get(x_15, 0); -x_18 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__2; -x_19 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__10; +x_18 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__2; +x_19 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__10; lean_inc(x_10); x_20 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_20, 0, x_10); lean_ctor_set(x_20, 1, x_18); lean_ctor_set(x_20, 2, x_19); -x_21 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__11; +x_21 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__11; lean_inc(x_10); lean_ctor_set_tag(x_11, 2); lean_ctor_set(x_11, 1, x_21); lean_ctor_set(x_11, 0, x_10); -x_22 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__12; +x_22 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__12; lean_inc(x_10); x_23 = l_Lean_Syntax_node1(x_10, x_22, x_11); lean_inc(x_10); x_24 = l_Lean_Syntax_node1(x_10, x_18, x_23); -x_25 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__9; +x_25 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__9; lean_inc_n(x_20, 5); lean_inc(x_10); x_26 = l_Lean_Syntax_node6(x_10, x_25, x_20, x_20, x_20, x_20, x_24, x_20); -x_27 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__15; +x_27 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__15; lean_inc(x_10); lean_ctor_set_tag(x_5, 2); lean_ctor_set(x_5, 1, x_27); lean_ctor_set(x_5, 0, x_10); -x_28 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__20; +x_28 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__20; lean_inc(x_13); lean_inc(x_17); x_29 = l_Lean_addMacroScope(x_17, x_28, x_13); x_30 = lean_box(0); -x_31 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__19; +x_31 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__19; lean_inc(x_10); x_32 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_32, 0, x_10); 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_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__17; +x_33 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__17; lean_inc(x_20); lean_inc(x_32); lean_inc(x_10); x_34 = l_Lean_Syntax_node2(x_10, x_33, x_32, x_20); -x_35 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__26; +x_35 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__26; lean_inc(x_10); x_36 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_36, 0, x_10); lean_ctor_set(x_36, 1, x_35); -x_37 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__31; +x_37 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__31; lean_inc(x_13); lean_inc(x_17); x_38 = l_Lean_addMacroScope(x_17, x_37, x_13); -x_39 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__30; -x_40 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__35; +x_39 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__30; +x_40 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__35; lean_inc(x_10); x_41 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_41, 0, x_10); lean_ctor_set(x_41, 1, x_39); lean_ctor_set(x_41, 2, x_38); lean_ctor_set(x_41, 3, x_40); -x_42 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__38; +x_42 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__38; lean_inc(x_10); x_43 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_43, 0, x_10); @@ -986,76 +1212,76 @@ lean_ctor_set(x_43, 1, x_42); x_44 = lean_box(0); lean_inc(x_1); x_45 = l_Lean_mkCIdentFrom(x_44, x_1, x_9); -x_46 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__37; +x_46 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__37; lean_inc(x_10); x_47 = l_Lean_Syntax_node2(x_10, x_46, x_43, x_45); lean_inc(x_10); x_48 = l_Lean_Syntax_node1(x_10, x_18, x_47); -x_49 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__28; +x_49 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__28; lean_inc(x_10); x_50 = l_Lean_Syntax_node2(x_10, x_49, x_41, x_48); -x_51 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__25; +x_51 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__25; lean_inc(x_10); x_52 = l_Lean_Syntax_node2(x_10, x_51, x_36, x_50); lean_inc(x_52); lean_inc(x_10); x_53 = l_Lean_Syntax_node1(x_10, x_18, x_52); -x_54 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__22; +x_54 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__22; lean_inc(x_20); lean_inc(x_10); x_55 = l_Lean_Syntax_node2(x_10, x_54, x_20, x_53); -x_56 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__41; +x_56 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__41; lean_inc(x_10); x_57 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_57, 0, x_10); lean_ctor_set(x_57, 1, x_56); -x_58 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__44; +x_58 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__44; lean_inc(x_10); x_59 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_59, 0, x_10); lean_ctor_set(x_59, 1, x_58); -x_60 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__47; +x_60 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__47; lean_inc(x_13); lean_inc(x_17); x_61 = l_Lean_addMacroScope(x_17, x_60, x_13); -x_62 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__46; +x_62 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__46; lean_inc(x_10); x_63 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_63, 0, x_10); lean_ctor_set(x_63, 1, x_62); lean_ctor_set(x_63, 2, x_61); lean_ctor_set(x_63, 3, x_30); -x_64 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__43; +x_64 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__43; lean_inc(x_10); x_65 = l_Lean_Syntax_node2(x_10, x_64, x_59, x_63); -x_66 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__50; +x_66 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__50; lean_inc(x_10); x_67 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_67, 0, x_10); lean_ctor_set(x_67, 1, x_66); -x_68 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__49; +x_68 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__49; lean_inc(x_10); x_69 = l_Lean_Syntax_node1(x_10, x_68, x_67); lean_inc(x_1); x_70 = l___private_Init_Meta_0__Lean_getEscapedNameParts_x3f(x_30, x_1); -x_71 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__53; +x_71 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__53; lean_inc_n(x_20, 2); lean_inc(x_10); x_72 = l_Lean_Syntax_node2(x_10, x_71, x_20, x_20); -x_73 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__56; +x_73 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__56; lean_inc(x_10); x_74 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_74, 0, x_10); lean_ctor_set(x_74, 1, x_73); -x_75 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__60; +x_75 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__60; lean_inc(x_20); lean_inc(x_10); x_76 = l_Lean_Syntax_node1(x_10, x_75, x_20); -x_77 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__66; +x_77 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__66; lean_inc(x_13); lean_inc(x_17); x_78 = l_Lean_addMacroScope(x_17, x_77, x_13); -x_79 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__65; +x_79 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__65; lean_inc(x_10); x_80 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_80, 0, x_10); @@ -1064,21 +1290,21 @@ lean_ctor_set(x_80, 2, x_78); lean_ctor_set(x_80, 3, x_30); lean_inc(x_10); x_81 = l_Lean_Syntax_node1(x_10, x_18, x_32); -x_82 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__63; +x_82 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__63; lean_inc(x_10); x_83 = l_Lean_Syntax_node2(x_10, x_82, x_80, x_81); -x_84 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__58; +x_84 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__58; lean_inc(x_76); lean_inc(x_10); x_85 = l_Lean_Syntax_node2(x_10, x_84, x_76, x_83); lean_inc(x_10); x_86 = l_Lean_Syntax_node1(x_10, x_18, x_85); -x_87 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__67; +x_87 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__67; lean_inc(x_10); x_88 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_88, 0, x_10); lean_ctor_set(x_88, 1, x_87); -x_89 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__55; +x_89 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__55; lean_inc(x_10); x_90 = l_Lean_Syntax_node3(x_10, x_89, x_74, x_86, x_88); lean_inc(x_10); @@ -1086,14 +1312,14 @@ x_91 = l_Lean_Syntax_node1(x_10, x_18, x_90); lean_inc_n(x_20, 5); lean_inc(x_10); x_92 = l_Lean_Syntax_node6(x_10, x_25, x_20, x_91, x_20, x_20, x_20, x_20); -x_93 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__68; +x_93 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__68; lean_inc(x_10); x_94 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_94, 0, x_10); lean_ctor_set(x_94, 1, x_93); -x_95 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__72; +x_95 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__72; x_96 = l_Lean_addMacroScope(x_17, x_95, x_13); -x_97 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__71; +x_97 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__71; lean_inc(x_10); x_98 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_98, 0, x_10); @@ -1104,33 +1330,33 @@ lean_inc(x_20); lean_inc(x_98); lean_inc(x_10); x_99 = l_Lean_Syntax_node2(x_10, x_33, x_98, x_20); -x_100 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__74; +x_100 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__74; lean_inc(x_20); lean_inc(x_10); x_101 = l_Lean_Syntax_node2(x_10, x_100, x_20, x_52); -x_102 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__69; +x_102 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__69; lean_inc(x_20); lean_inc(x_101); lean_inc(x_10); x_103 = l_Lean_Syntax_node4(x_10, x_102, x_94, x_99, x_101, x_20); -x_104 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__7; +x_104 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__7; lean_inc(x_10); x_105 = l_Lean_Syntax_node2(x_10, x_104, x_92, x_103); lean_inc_n(x_20, 6); lean_inc(x_10); x_106 = l_Lean_Syntax_node6(x_10, x_25, x_20, x_20, x_20, x_20, x_20, x_20); -x_107 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__75; +x_107 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__75; lean_inc(x_10); x_108 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_108, 0, x_10); lean_ctor_set(x_108, 1, x_107); -x_109 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__40; +x_109 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__40; lean_inc(x_20); lean_inc(x_72); lean_inc(x_57); lean_inc(x_10); x_110 = l_Lean_Syntax_node4(x_10, x_109, x_57, x_98, x_72, x_20); -x_111 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__76; +x_111 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__76; lean_inc_n(x_20, 2); lean_inc(x_10); x_112 = l_Lean_Syntax_node6(x_10, x_111, x_76, x_108, x_20, x_20, x_101, x_110); @@ -1147,7 +1373,7 @@ x_116 = l_Lean_Syntax_node2(x_10, x_49, x_65, x_115); lean_inc(x_20); lean_inc(x_10); x_117 = l_Lean_Syntax_node4(x_10, x_109, x_57, x_116, x_72, x_20); -x_118 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__14; +x_118 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__14; lean_inc(x_10); x_119 = l_Lean_Syntax_node5(x_10, x_118, x_5, x_34, x_55, x_117, x_20); lean_inc(x_10); @@ -1164,7 +1390,7 @@ x_122 = lean_ctor_get(x_70, 0); lean_inc(x_122); lean_dec(x_70); x_123 = l_String_intercalate(x_58, x_122); -x_124 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__79; +x_124 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__79; x_125 = lean_string_append(x_124, x_123); lean_dec(x_123); x_126 = lean_box(2); @@ -1173,7 +1399,7 @@ x_128 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_128, 0, x_127); lean_ctor_set(x_128, 1, x_30); x_129 = lean_array_mk(x_128); -x_130 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__78; +x_130 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__78; x_131 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_131, 0, x_126); lean_ctor_set(x_131, 1, x_130); @@ -1185,7 +1411,7 @@ x_133 = l_Lean_Syntax_node2(x_10, x_49, x_65, x_132); lean_inc(x_20); lean_inc(x_10); x_134 = l_Lean_Syntax_node4(x_10, x_109, x_57, x_133, x_72, x_20); -x_135 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__14; +x_135 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__14; lean_inc(x_10); x_136 = l_Lean_Syntax_node5(x_10, x_135, x_5, x_34, x_55, x_134, x_20); lean_inc(x_10); @@ -1203,67 +1429,67 @@ x_140 = lean_ctor_get(x_15, 1); lean_inc(x_140); lean_inc(x_139); lean_dec(x_15); -x_141 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__2; -x_142 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__10; +x_141 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__2; +x_142 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__10; lean_inc(x_10); x_143 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_143, 0, x_10); lean_ctor_set(x_143, 1, x_141); lean_ctor_set(x_143, 2, x_142); -x_144 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__11; +x_144 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__11; lean_inc(x_10); lean_ctor_set_tag(x_11, 2); lean_ctor_set(x_11, 1, x_144); lean_ctor_set(x_11, 0, x_10); -x_145 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__12; +x_145 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__12; lean_inc(x_10); x_146 = l_Lean_Syntax_node1(x_10, x_145, x_11); lean_inc(x_10); x_147 = l_Lean_Syntax_node1(x_10, x_141, x_146); -x_148 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__9; +x_148 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__9; lean_inc_n(x_143, 5); lean_inc(x_10); x_149 = l_Lean_Syntax_node6(x_10, x_148, x_143, x_143, x_143, x_143, x_147, x_143); -x_150 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__15; +x_150 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__15; lean_inc(x_10); lean_ctor_set_tag(x_5, 2); lean_ctor_set(x_5, 1, x_150); lean_ctor_set(x_5, 0, x_10); -x_151 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__20; +x_151 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__20; lean_inc(x_13); lean_inc(x_139); x_152 = l_Lean_addMacroScope(x_139, x_151, x_13); x_153 = lean_box(0); -x_154 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__19; +x_154 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__19; lean_inc(x_10); x_155 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_155, 0, x_10); lean_ctor_set(x_155, 1, x_154); lean_ctor_set(x_155, 2, x_152); lean_ctor_set(x_155, 3, x_153); -x_156 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__17; +x_156 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__17; lean_inc(x_143); lean_inc(x_155); lean_inc(x_10); x_157 = l_Lean_Syntax_node2(x_10, x_156, x_155, x_143); -x_158 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__26; +x_158 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__26; lean_inc(x_10); x_159 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_159, 0, x_10); lean_ctor_set(x_159, 1, x_158); -x_160 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__31; +x_160 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__31; lean_inc(x_13); lean_inc(x_139); x_161 = l_Lean_addMacroScope(x_139, x_160, x_13); -x_162 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__30; -x_163 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__35; +x_162 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__30; +x_163 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__35; lean_inc(x_10); x_164 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_164, 0, x_10); lean_ctor_set(x_164, 1, x_162); lean_ctor_set(x_164, 2, x_161); lean_ctor_set(x_164, 3, x_163); -x_165 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__38; +x_165 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__38; lean_inc(x_10); x_166 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_166, 0, x_10); @@ -1271,76 +1497,76 @@ lean_ctor_set(x_166, 1, x_165); x_167 = lean_box(0); lean_inc(x_1); x_168 = l_Lean_mkCIdentFrom(x_167, x_1, x_9); -x_169 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__37; +x_169 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__37; lean_inc(x_10); x_170 = l_Lean_Syntax_node2(x_10, x_169, x_166, x_168); lean_inc(x_10); x_171 = l_Lean_Syntax_node1(x_10, x_141, x_170); -x_172 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__28; +x_172 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__28; lean_inc(x_10); x_173 = l_Lean_Syntax_node2(x_10, x_172, x_164, x_171); -x_174 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__25; +x_174 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__25; lean_inc(x_10); x_175 = l_Lean_Syntax_node2(x_10, x_174, x_159, x_173); lean_inc(x_175); lean_inc(x_10); x_176 = l_Lean_Syntax_node1(x_10, x_141, x_175); -x_177 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__22; +x_177 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__22; lean_inc(x_143); lean_inc(x_10); x_178 = l_Lean_Syntax_node2(x_10, x_177, x_143, x_176); -x_179 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__41; +x_179 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__41; lean_inc(x_10); x_180 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_180, 0, x_10); lean_ctor_set(x_180, 1, x_179); -x_181 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__44; +x_181 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__44; lean_inc(x_10); x_182 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_182, 0, x_10); lean_ctor_set(x_182, 1, x_181); -x_183 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__47; +x_183 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__47; lean_inc(x_13); lean_inc(x_139); x_184 = l_Lean_addMacroScope(x_139, x_183, x_13); -x_185 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__46; +x_185 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__46; lean_inc(x_10); x_186 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_186, 0, x_10); lean_ctor_set(x_186, 1, x_185); lean_ctor_set(x_186, 2, x_184); lean_ctor_set(x_186, 3, x_153); -x_187 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__43; +x_187 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__43; lean_inc(x_10); x_188 = l_Lean_Syntax_node2(x_10, x_187, x_182, x_186); -x_189 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__50; +x_189 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__50; lean_inc(x_10); x_190 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_190, 0, x_10); lean_ctor_set(x_190, 1, x_189); -x_191 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__49; +x_191 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__49; lean_inc(x_10); x_192 = l_Lean_Syntax_node1(x_10, x_191, x_190); lean_inc(x_1); x_193 = l___private_Init_Meta_0__Lean_getEscapedNameParts_x3f(x_153, x_1); -x_194 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__53; +x_194 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__53; lean_inc_n(x_143, 2); lean_inc(x_10); x_195 = l_Lean_Syntax_node2(x_10, x_194, x_143, x_143); -x_196 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__56; +x_196 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__56; lean_inc(x_10); x_197 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_197, 0, x_10); lean_ctor_set(x_197, 1, x_196); -x_198 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__60; +x_198 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__60; lean_inc(x_143); lean_inc(x_10); x_199 = l_Lean_Syntax_node1(x_10, x_198, x_143); -x_200 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__66; +x_200 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__66; lean_inc(x_13); lean_inc(x_139); x_201 = l_Lean_addMacroScope(x_139, x_200, x_13); -x_202 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__65; +x_202 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__65; lean_inc(x_10); x_203 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_203, 0, x_10); @@ -1349,21 +1575,21 @@ lean_ctor_set(x_203, 2, x_201); lean_ctor_set(x_203, 3, x_153); lean_inc(x_10); x_204 = l_Lean_Syntax_node1(x_10, x_141, x_155); -x_205 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__63; +x_205 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__63; lean_inc(x_10); x_206 = l_Lean_Syntax_node2(x_10, x_205, x_203, x_204); -x_207 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__58; +x_207 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__58; lean_inc(x_199); lean_inc(x_10); x_208 = l_Lean_Syntax_node2(x_10, x_207, x_199, x_206); lean_inc(x_10); x_209 = l_Lean_Syntax_node1(x_10, x_141, x_208); -x_210 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__67; +x_210 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__67; lean_inc(x_10); x_211 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_211, 0, x_10); lean_ctor_set(x_211, 1, x_210); -x_212 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__55; +x_212 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__55; lean_inc(x_10); x_213 = l_Lean_Syntax_node3(x_10, x_212, x_197, x_209, x_211); lean_inc(x_10); @@ -1371,14 +1597,14 @@ x_214 = l_Lean_Syntax_node1(x_10, x_141, x_213); lean_inc_n(x_143, 5); lean_inc(x_10); x_215 = l_Lean_Syntax_node6(x_10, x_148, x_143, x_214, x_143, x_143, x_143, x_143); -x_216 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__68; +x_216 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__68; lean_inc(x_10); x_217 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_217, 0, x_10); lean_ctor_set(x_217, 1, x_216); -x_218 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__72; +x_218 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__72; x_219 = l_Lean_addMacroScope(x_139, x_218, x_13); -x_220 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__71; +x_220 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__71; lean_inc(x_10); x_221 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_221, 0, x_10); @@ -1389,33 +1615,33 @@ lean_inc(x_143); lean_inc(x_221); lean_inc(x_10); x_222 = l_Lean_Syntax_node2(x_10, x_156, x_221, x_143); -x_223 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__74; +x_223 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__74; lean_inc(x_143); lean_inc(x_10); x_224 = l_Lean_Syntax_node2(x_10, x_223, x_143, x_175); -x_225 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__69; +x_225 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__69; lean_inc(x_143); lean_inc(x_224); lean_inc(x_10); x_226 = l_Lean_Syntax_node4(x_10, x_225, x_217, x_222, x_224, x_143); -x_227 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__7; +x_227 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__7; lean_inc(x_10); x_228 = l_Lean_Syntax_node2(x_10, x_227, x_215, x_226); lean_inc_n(x_143, 6); lean_inc(x_10); x_229 = l_Lean_Syntax_node6(x_10, x_148, x_143, x_143, x_143, x_143, x_143, x_143); -x_230 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__75; +x_230 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__75; lean_inc(x_10); x_231 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_231, 0, x_10); lean_ctor_set(x_231, 1, x_230); -x_232 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__40; +x_232 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__40; lean_inc(x_143); lean_inc(x_195); lean_inc(x_180); lean_inc(x_10); x_233 = l_Lean_Syntax_node4(x_10, x_232, x_180, x_221, x_195, x_143); -x_234 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__76; +x_234 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__76; lean_inc_n(x_143, 2); lean_inc(x_10); x_235 = l_Lean_Syntax_node6(x_10, x_234, x_199, x_231, x_143, x_143, x_224, x_233); @@ -1432,7 +1658,7 @@ x_239 = l_Lean_Syntax_node2(x_10, x_172, x_188, x_238); lean_inc(x_143); lean_inc(x_10); x_240 = l_Lean_Syntax_node4(x_10, x_232, x_180, x_239, x_195, x_143); -x_241 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__14; +x_241 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__14; lean_inc(x_10); x_242 = l_Lean_Syntax_node5(x_10, x_241, x_5, x_157, x_178, x_240, x_143); lean_inc(x_10); @@ -1451,7 +1677,7 @@ x_246 = lean_ctor_get(x_193, 0); lean_inc(x_246); lean_dec(x_193); x_247 = l_String_intercalate(x_181, x_246); -x_248 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__79; +x_248 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__79; x_249 = lean_string_append(x_248, x_247); lean_dec(x_247); x_250 = lean_box(2); @@ -1460,7 +1686,7 @@ x_252 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_252, 0, x_251); lean_ctor_set(x_252, 1, x_153); x_253 = lean_array_mk(x_252); -x_254 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__78; +x_254 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__78; x_255 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_255, 0, x_250); lean_ctor_set(x_255, 1, x_254); @@ -1472,7 +1698,7 @@ x_257 = l_Lean_Syntax_node2(x_10, x_172, x_188, x_256); lean_inc(x_143); lean_inc(x_10); x_258 = l_Lean_Syntax_node4(x_10, x_232, x_180, x_257, x_195, x_143); -x_259 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__14; +x_259 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__14; lean_inc(x_10); x_260 = l_Lean_Syntax_node5(x_10, x_259, x_5, x_157, x_178, x_258, x_143); lean_inc(x_10); @@ -1506,67 +1732,67 @@ if (lean_is_exclusive(x_266)) { lean_dec_ref(x_266); x_269 = lean_box(0); } -x_270 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__2; -x_271 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__10; +x_270 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__2; +x_271 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__10; lean_inc(x_10); x_272 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_272, 0, x_10); lean_ctor_set(x_272, 1, x_270); lean_ctor_set(x_272, 2, x_271); -x_273 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__11; +x_273 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__11; lean_inc(x_10); x_274 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_274, 0, x_10); lean_ctor_set(x_274, 1, x_273); -x_275 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__12; +x_275 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__12; lean_inc(x_10); x_276 = l_Lean_Syntax_node1(x_10, x_275, x_274); lean_inc(x_10); x_277 = l_Lean_Syntax_node1(x_10, x_270, x_276); -x_278 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__9; +x_278 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__9; lean_inc_n(x_272, 5); lean_inc(x_10); x_279 = l_Lean_Syntax_node6(x_10, x_278, x_272, x_272, x_272, x_272, x_277, x_272); -x_280 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__15; +x_280 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__15; lean_inc(x_10); lean_ctor_set_tag(x_5, 2); lean_ctor_set(x_5, 1, x_280); lean_ctor_set(x_5, 0, x_10); -x_281 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__20; +x_281 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__20; lean_inc(x_264); lean_inc(x_267); x_282 = l_Lean_addMacroScope(x_267, x_281, x_264); x_283 = lean_box(0); -x_284 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__19; +x_284 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__19; lean_inc(x_10); x_285 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_285, 0, x_10); lean_ctor_set(x_285, 1, x_284); lean_ctor_set(x_285, 2, x_282); lean_ctor_set(x_285, 3, x_283); -x_286 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__17; +x_286 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__17; lean_inc(x_272); lean_inc(x_285); lean_inc(x_10); x_287 = l_Lean_Syntax_node2(x_10, x_286, x_285, x_272); -x_288 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__26; +x_288 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__26; lean_inc(x_10); x_289 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_289, 0, x_10); lean_ctor_set(x_289, 1, x_288); -x_290 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__31; +x_290 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__31; lean_inc(x_264); lean_inc(x_267); x_291 = l_Lean_addMacroScope(x_267, x_290, x_264); -x_292 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__30; -x_293 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__35; +x_292 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__30; +x_293 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__35; lean_inc(x_10); x_294 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_294, 0, x_10); lean_ctor_set(x_294, 1, x_292); lean_ctor_set(x_294, 2, x_291); lean_ctor_set(x_294, 3, x_293); -x_295 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__38; +x_295 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__38; lean_inc(x_10); x_296 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_296, 0, x_10); @@ -1574,76 +1800,76 @@ lean_ctor_set(x_296, 1, x_295); x_297 = lean_box(0); lean_inc(x_1); x_298 = l_Lean_mkCIdentFrom(x_297, x_1, x_9); -x_299 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__37; +x_299 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__37; lean_inc(x_10); x_300 = l_Lean_Syntax_node2(x_10, x_299, x_296, x_298); lean_inc(x_10); x_301 = l_Lean_Syntax_node1(x_10, x_270, x_300); -x_302 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__28; +x_302 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__28; lean_inc(x_10); x_303 = l_Lean_Syntax_node2(x_10, x_302, x_294, x_301); -x_304 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__25; +x_304 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__25; lean_inc(x_10); x_305 = l_Lean_Syntax_node2(x_10, x_304, x_289, x_303); lean_inc(x_305); lean_inc(x_10); x_306 = l_Lean_Syntax_node1(x_10, x_270, x_305); -x_307 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__22; +x_307 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__22; lean_inc(x_272); lean_inc(x_10); x_308 = l_Lean_Syntax_node2(x_10, x_307, x_272, x_306); -x_309 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__41; +x_309 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__41; lean_inc(x_10); x_310 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_310, 0, x_10); lean_ctor_set(x_310, 1, x_309); -x_311 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__44; +x_311 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__44; lean_inc(x_10); x_312 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_312, 0, x_10); lean_ctor_set(x_312, 1, x_311); -x_313 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__47; +x_313 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__47; lean_inc(x_264); lean_inc(x_267); x_314 = l_Lean_addMacroScope(x_267, x_313, x_264); -x_315 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__46; +x_315 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__46; lean_inc(x_10); x_316 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_316, 0, x_10); lean_ctor_set(x_316, 1, x_315); lean_ctor_set(x_316, 2, x_314); lean_ctor_set(x_316, 3, x_283); -x_317 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__43; +x_317 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__43; lean_inc(x_10); x_318 = l_Lean_Syntax_node2(x_10, x_317, x_312, x_316); -x_319 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__50; +x_319 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__50; lean_inc(x_10); x_320 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_320, 0, x_10); lean_ctor_set(x_320, 1, x_319); -x_321 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__49; +x_321 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__49; lean_inc(x_10); x_322 = l_Lean_Syntax_node1(x_10, x_321, x_320); lean_inc(x_1); x_323 = l___private_Init_Meta_0__Lean_getEscapedNameParts_x3f(x_283, x_1); -x_324 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__53; +x_324 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__53; lean_inc_n(x_272, 2); lean_inc(x_10); x_325 = l_Lean_Syntax_node2(x_10, x_324, x_272, x_272); -x_326 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__56; +x_326 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__56; lean_inc(x_10); x_327 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_327, 0, x_10); lean_ctor_set(x_327, 1, x_326); -x_328 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__60; +x_328 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__60; lean_inc(x_272); lean_inc(x_10); x_329 = l_Lean_Syntax_node1(x_10, x_328, x_272); -x_330 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__66; +x_330 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__66; lean_inc(x_264); lean_inc(x_267); x_331 = l_Lean_addMacroScope(x_267, x_330, x_264); -x_332 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__65; +x_332 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__65; lean_inc(x_10); x_333 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_333, 0, x_10); @@ -1652,21 +1878,21 @@ lean_ctor_set(x_333, 2, x_331); lean_ctor_set(x_333, 3, x_283); lean_inc(x_10); x_334 = l_Lean_Syntax_node1(x_10, x_270, x_285); -x_335 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__63; +x_335 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__63; lean_inc(x_10); x_336 = l_Lean_Syntax_node2(x_10, x_335, x_333, x_334); -x_337 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__58; +x_337 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__58; lean_inc(x_329); lean_inc(x_10); x_338 = l_Lean_Syntax_node2(x_10, x_337, x_329, x_336); lean_inc(x_10); x_339 = l_Lean_Syntax_node1(x_10, x_270, x_338); -x_340 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__67; +x_340 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__67; lean_inc(x_10); x_341 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_341, 0, x_10); lean_ctor_set(x_341, 1, x_340); -x_342 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__55; +x_342 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__55; lean_inc(x_10); x_343 = l_Lean_Syntax_node3(x_10, x_342, x_327, x_339, x_341); lean_inc(x_10); @@ -1674,14 +1900,14 @@ x_344 = l_Lean_Syntax_node1(x_10, x_270, x_343); lean_inc_n(x_272, 5); lean_inc(x_10); x_345 = l_Lean_Syntax_node6(x_10, x_278, x_272, x_344, x_272, x_272, x_272, x_272); -x_346 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__68; +x_346 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__68; lean_inc(x_10); x_347 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_347, 0, x_10); lean_ctor_set(x_347, 1, x_346); -x_348 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__72; +x_348 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__72; x_349 = l_Lean_addMacroScope(x_267, x_348, x_264); -x_350 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__71; +x_350 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__71; lean_inc(x_10); x_351 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_351, 0, x_10); @@ -1692,33 +1918,33 @@ lean_inc(x_272); lean_inc(x_351); lean_inc(x_10); x_352 = l_Lean_Syntax_node2(x_10, x_286, x_351, x_272); -x_353 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__74; +x_353 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__74; lean_inc(x_272); lean_inc(x_10); x_354 = l_Lean_Syntax_node2(x_10, x_353, x_272, x_305); -x_355 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__69; +x_355 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__69; lean_inc(x_272); lean_inc(x_354); lean_inc(x_10); x_356 = l_Lean_Syntax_node4(x_10, x_355, x_347, x_352, x_354, x_272); -x_357 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__7; +x_357 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__7; lean_inc(x_10); x_358 = l_Lean_Syntax_node2(x_10, x_357, x_345, x_356); lean_inc_n(x_272, 6); lean_inc(x_10); x_359 = l_Lean_Syntax_node6(x_10, x_278, x_272, x_272, x_272, x_272, x_272, x_272); -x_360 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__75; +x_360 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__75; lean_inc(x_10); x_361 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_361, 0, x_10); lean_ctor_set(x_361, 1, x_360); -x_362 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__40; +x_362 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__40; lean_inc(x_272); lean_inc(x_325); lean_inc(x_310); lean_inc(x_10); x_363 = l_Lean_Syntax_node4(x_10, x_362, x_310, x_351, x_325, x_272); -x_364 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__76; +x_364 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__76; lean_inc_n(x_272, 2); lean_inc(x_10); x_365 = l_Lean_Syntax_node6(x_10, x_364, x_329, x_361, x_272, x_272, x_354, x_363); @@ -1735,7 +1961,7 @@ x_369 = l_Lean_Syntax_node2(x_10, x_302, x_318, x_368); lean_inc(x_272); lean_inc(x_10); x_370 = l_Lean_Syntax_node4(x_10, x_362, x_310, x_369, x_325, x_272); -x_371 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__14; +x_371 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__14; lean_inc(x_10); x_372 = l_Lean_Syntax_node5(x_10, x_371, x_5, x_287, x_308, x_370, x_272); lean_inc(x_10); @@ -1758,7 +1984,7 @@ x_376 = lean_ctor_get(x_323, 0); lean_inc(x_376); lean_dec(x_323); x_377 = l_String_intercalate(x_311, x_376); -x_378 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__79; +x_378 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__79; x_379 = lean_string_append(x_378, x_377); lean_dec(x_377); x_380 = lean_box(2); @@ -1767,7 +1993,7 @@ x_382 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_382, 0, x_381); lean_ctor_set(x_382, 1, x_283); x_383 = lean_array_mk(x_382); -x_384 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__78; +x_384 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__78; x_385 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_385, 0, x_380); lean_ctor_set(x_385, 1, x_384); @@ -1779,7 +2005,7 @@ x_387 = l_Lean_Syntax_node2(x_10, x_302, x_318, x_386); lean_inc(x_272); lean_inc(x_10); x_388 = l_Lean_Syntax_node4(x_10, x_362, x_310, x_387, x_325, x_272); -x_389 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__14; +x_389 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__14; lean_inc(x_10); x_390 = l_Lean_Syntax_node5(x_10, x_389, x_5, x_287, x_308, x_388, x_272); lean_inc(x_10); @@ -1833,14 +2059,14 @@ if (lean_is_exclusive(x_402)) { lean_dec_ref(x_402); x_405 = lean_box(0); } -x_406 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__2; -x_407 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__10; +x_406 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__2; +x_407 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__10; lean_inc(x_397); x_408 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_408, 0, x_397); lean_ctor_set(x_408, 1, x_406); lean_ctor_set(x_408, 2, x_407); -x_409 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__11; +x_409 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__11; lean_inc(x_397); if (lean_is_scalar(x_401)) { x_410 = lean_alloc_ctor(2, 2, 0); @@ -1850,55 +2076,55 @@ if (lean_is_scalar(x_401)) { } lean_ctor_set(x_410, 0, x_397); lean_ctor_set(x_410, 1, x_409); -x_411 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__12; +x_411 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__12; lean_inc(x_397); x_412 = l_Lean_Syntax_node1(x_397, x_411, x_410); lean_inc(x_397); x_413 = l_Lean_Syntax_node1(x_397, x_406, x_412); -x_414 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__9; +x_414 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__9; lean_inc_n(x_408, 5); lean_inc(x_397); x_415 = l_Lean_Syntax_node6(x_397, x_414, x_408, x_408, x_408, x_408, x_413, x_408); -x_416 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__15; +x_416 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__15; lean_inc(x_397); x_417 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_417, 0, x_397); lean_ctor_set(x_417, 1, x_416); -x_418 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__20; +x_418 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__20; lean_inc(x_399); lean_inc(x_403); x_419 = l_Lean_addMacroScope(x_403, x_418, x_399); x_420 = lean_box(0); -x_421 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__19; +x_421 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__19; lean_inc(x_397); x_422 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_422, 0, x_397); lean_ctor_set(x_422, 1, x_421); lean_ctor_set(x_422, 2, x_419); lean_ctor_set(x_422, 3, x_420); -x_423 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__17; +x_423 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__17; lean_inc(x_408); lean_inc(x_422); lean_inc(x_397); x_424 = l_Lean_Syntax_node2(x_397, x_423, x_422, x_408); -x_425 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__26; +x_425 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__26; lean_inc(x_397); x_426 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_426, 0, x_397); lean_ctor_set(x_426, 1, x_425); -x_427 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__31; +x_427 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__31; lean_inc(x_399); lean_inc(x_403); x_428 = l_Lean_addMacroScope(x_403, x_427, x_399); -x_429 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__30; -x_430 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__35; +x_429 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__30; +x_430 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__35; lean_inc(x_397); x_431 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_431, 0, x_397); lean_ctor_set(x_431, 1, x_429); lean_ctor_set(x_431, 2, x_428); lean_ctor_set(x_431, 3, x_430); -x_432 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__38; +x_432 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__38; lean_inc(x_397); x_433 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_433, 0, x_397); @@ -1906,76 +2132,76 @@ lean_ctor_set(x_433, 1, x_432); x_434 = lean_box(0); lean_inc(x_1); x_435 = l_Lean_mkCIdentFrom(x_434, x_1, x_396); -x_436 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__37; +x_436 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__37; lean_inc(x_397); x_437 = l_Lean_Syntax_node2(x_397, x_436, x_433, x_435); lean_inc(x_397); x_438 = l_Lean_Syntax_node1(x_397, x_406, x_437); -x_439 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__28; +x_439 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__28; lean_inc(x_397); x_440 = l_Lean_Syntax_node2(x_397, x_439, x_431, x_438); -x_441 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__25; +x_441 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__25; lean_inc(x_397); x_442 = l_Lean_Syntax_node2(x_397, x_441, x_426, x_440); lean_inc(x_442); lean_inc(x_397); x_443 = l_Lean_Syntax_node1(x_397, x_406, x_442); -x_444 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__22; +x_444 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__22; lean_inc(x_408); lean_inc(x_397); x_445 = l_Lean_Syntax_node2(x_397, x_444, x_408, x_443); -x_446 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__41; +x_446 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__41; lean_inc(x_397); x_447 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_447, 0, x_397); lean_ctor_set(x_447, 1, x_446); -x_448 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__44; +x_448 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__44; lean_inc(x_397); x_449 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_449, 0, x_397); lean_ctor_set(x_449, 1, x_448); -x_450 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__47; +x_450 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__47; lean_inc(x_399); lean_inc(x_403); x_451 = l_Lean_addMacroScope(x_403, x_450, x_399); -x_452 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__46; +x_452 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__46; lean_inc(x_397); x_453 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_453, 0, x_397); lean_ctor_set(x_453, 1, x_452); lean_ctor_set(x_453, 2, x_451); lean_ctor_set(x_453, 3, x_420); -x_454 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__43; +x_454 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__43; lean_inc(x_397); x_455 = l_Lean_Syntax_node2(x_397, x_454, x_449, x_453); -x_456 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__50; +x_456 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__50; lean_inc(x_397); x_457 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_457, 0, x_397); lean_ctor_set(x_457, 1, x_456); -x_458 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__49; +x_458 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__49; lean_inc(x_397); x_459 = l_Lean_Syntax_node1(x_397, x_458, x_457); lean_inc(x_1); x_460 = l___private_Init_Meta_0__Lean_getEscapedNameParts_x3f(x_420, x_1); -x_461 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__53; +x_461 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__53; lean_inc_n(x_408, 2); lean_inc(x_397); x_462 = l_Lean_Syntax_node2(x_397, x_461, x_408, x_408); -x_463 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__56; +x_463 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__56; lean_inc(x_397); x_464 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_464, 0, x_397); lean_ctor_set(x_464, 1, x_463); -x_465 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__60; +x_465 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__60; lean_inc(x_408); lean_inc(x_397); x_466 = l_Lean_Syntax_node1(x_397, x_465, x_408); -x_467 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__66; +x_467 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__66; lean_inc(x_399); lean_inc(x_403); x_468 = l_Lean_addMacroScope(x_403, x_467, x_399); -x_469 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__65; +x_469 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__65; lean_inc(x_397); x_470 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_470, 0, x_397); @@ -1984,21 +2210,21 @@ lean_ctor_set(x_470, 2, x_468); lean_ctor_set(x_470, 3, x_420); lean_inc(x_397); x_471 = l_Lean_Syntax_node1(x_397, x_406, x_422); -x_472 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__63; +x_472 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__63; lean_inc(x_397); x_473 = l_Lean_Syntax_node2(x_397, x_472, x_470, x_471); -x_474 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__58; +x_474 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__58; lean_inc(x_466); lean_inc(x_397); x_475 = l_Lean_Syntax_node2(x_397, x_474, x_466, x_473); lean_inc(x_397); x_476 = l_Lean_Syntax_node1(x_397, x_406, x_475); -x_477 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__67; +x_477 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__67; lean_inc(x_397); x_478 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_478, 0, x_397); lean_ctor_set(x_478, 1, x_477); -x_479 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__55; +x_479 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__55; lean_inc(x_397); x_480 = l_Lean_Syntax_node3(x_397, x_479, x_464, x_476, x_478); lean_inc(x_397); @@ -2006,14 +2232,14 @@ x_481 = l_Lean_Syntax_node1(x_397, x_406, x_480); lean_inc_n(x_408, 5); lean_inc(x_397); x_482 = l_Lean_Syntax_node6(x_397, x_414, x_408, x_481, x_408, x_408, x_408, x_408); -x_483 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__68; +x_483 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__68; lean_inc(x_397); x_484 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_484, 0, x_397); lean_ctor_set(x_484, 1, x_483); -x_485 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__72; +x_485 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__72; x_486 = l_Lean_addMacroScope(x_403, x_485, x_399); -x_487 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__71; +x_487 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__71; lean_inc(x_397); x_488 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_488, 0, x_397); @@ -2024,33 +2250,33 @@ lean_inc(x_408); lean_inc(x_488); lean_inc(x_397); x_489 = l_Lean_Syntax_node2(x_397, x_423, x_488, x_408); -x_490 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__74; +x_490 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__74; lean_inc(x_408); lean_inc(x_397); x_491 = l_Lean_Syntax_node2(x_397, x_490, x_408, x_442); -x_492 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__69; +x_492 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__69; lean_inc(x_408); lean_inc(x_491); lean_inc(x_397); x_493 = l_Lean_Syntax_node4(x_397, x_492, x_484, x_489, x_491, x_408); -x_494 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__7; +x_494 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__7; lean_inc(x_397); x_495 = l_Lean_Syntax_node2(x_397, x_494, x_482, x_493); lean_inc_n(x_408, 6); lean_inc(x_397); x_496 = l_Lean_Syntax_node6(x_397, x_414, x_408, x_408, x_408, x_408, x_408, x_408); -x_497 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__75; +x_497 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__75; lean_inc(x_397); x_498 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_498, 0, x_397); lean_ctor_set(x_498, 1, x_497); -x_499 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__40; +x_499 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__40; lean_inc(x_408); lean_inc(x_462); lean_inc(x_447); lean_inc(x_397); x_500 = l_Lean_Syntax_node4(x_397, x_499, x_447, x_488, x_462, x_408); -x_501 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__76; +x_501 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__76; lean_inc_n(x_408, 2); lean_inc(x_397); x_502 = l_Lean_Syntax_node6(x_397, x_501, x_466, x_498, x_408, x_408, x_491, x_500); @@ -2067,7 +2293,7 @@ x_506 = l_Lean_Syntax_node2(x_397, x_439, x_455, x_505); lean_inc(x_408); lean_inc(x_397); x_507 = l_Lean_Syntax_node4(x_397, x_499, x_447, x_506, x_462, x_408); -x_508 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__14; +x_508 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__14; lean_inc(x_397); x_509 = l_Lean_Syntax_node5(x_397, x_508, x_417, x_424, x_445, x_507, x_408); lean_inc(x_397); @@ -2090,7 +2316,7 @@ x_513 = lean_ctor_get(x_460, 0); lean_inc(x_513); lean_dec(x_460); x_514 = l_String_intercalate(x_448, x_513); -x_515 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__79; +x_515 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__79; x_516 = lean_string_append(x_515, x_514); lean_dec(x_514); x_517 = lean_box(2); @@ -2099,7 +2325,7 @@ x_519 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_519, 0, x_518); lean_ctor_set(x_519, 1, x_420); x_520 = lean_array_mk(x_519); -x_521 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__78; +x_521 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__78; x_522 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_522, 0, x_517); lean_ctor_set(x_522, 1, x_521); @@ -2111,7 +2337,7 @@ x_524 = l_Lean_Syntax_node2(x_397, x_439, x_455, x_523); lean_inc(x_408); lean_inc(x_397); x_525 = l_Lean_Syntax_node4(x_397, x_499, x_447, x_524, x_462, x_408); -x_526 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__14; +x_526 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__14; lean_inc(x_397); x_527 = l_Lean_Syntax_node5(x_397, x_526, x_417, x_424, x_445, x_525, x_408); lean_inc(x_397); @@ -2129,7 +2355,7 @@ return x_530; } } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__2___closed__1() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__2___closed__1() { _start: { lean_object* x_1; lean_object* x_2; @@ -2139,11 +2365,11 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___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_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___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; -x_6 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___boxed), 4, 1); +x_6 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___boxed), 4, 1); lean_closure_set(x_6, 0, x_1); lean_inc(x_4); lean_inc(x_3); @@ -2166,7 +2392,7 @@ if (x_11 == 0) lean_object* x_12; lean_object* x_13; x_12 = lean_ctor_get(x_10, 0); lean_dec(x_12); -x_13 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__2___closed__1; +x_13 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__2___closed__1; lean_ctor_set(x_10, 0, x_13); return x_10; } @@ -2176,7 +2402,7 @@ lean_object* x_14; lean_object* x_15; lean_object* x_16; x_14 = lean_ctor_get(x_10, 1); lean_inc(x_14); lean_dec(x_10); -x_15 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__2___closed__1; +x_15 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__2___closed__1; x_16 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_16, 0, x_15); lean_ctor_set(x_16, 1, x_14); @@ -2232,7 +2458,7 @@ return x_24; } } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__1() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___closed__1() { _start: { lean_object* x_1; @@ -2240,16 +2466,16 @@ x_1 = lean_mk_string_unchecked("", 0, 0); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__2() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__1; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__3() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___closed__3() { _start: { lean_object* x_1; @@ -2257,16 +2483,16 @@ x_1 = lean_mk_string_unchecked(" has universe level parameters", 30, 30); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__4() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__3; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___closed__3; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___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) { _start: { uint8_t x_8; @@ -2288,7 +2514,7 @@ lean_dec(x_4); x_10 = lean_array_uget(x_1, x_3); lean_inc(x_5); lean_inc(x_10); -x_11 = l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9(x_10, x_5, x_6, x_7); +x_11 = l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1(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; uint8_t x_15; @@ -2307,15 +2533,15 @@ lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean x_16 = lean_box(0); x_17 = l_Lean_Expr_const___override(x_10, x_16); x_18 = l_Lean_MessageData_ofExpr(x_17); -x_19 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__2; +x_19 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___closed__2; x_20 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_20, 0, x_19); lean_ctor_set(x_20, 1, x_18); -x_21 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__4; +x_21 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___closed__4; x_22 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_22, 0, x_20); lean_ctor_set(x_22, 1, x_21); -x_23 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_22, x_5, x_6, x_13); +x_23 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__7(x_22, x_5, x_6, x_13); lean_dec(x_6); x_24 = !lean_is_exclusive(x_23); if (x_24 == 0) @@ -2342,7 +2568,7 @@ lean_object* x_28; lean_object* x_29; x_28 = lean_box(0); lean_inc(x_6); lean_inc(x_5); -x_29 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__2(x_10, x_28, x_5, x_6, x_13); +x_29 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__2(x_10, x_28, x_5, x_6, x_13); if (lean_obj_tag(x_29) == 0) { lean_object* x_30; @@ -2458,7 +2684,7 @@ size_t x_5; size_t x_6; lean_object* x_7; lean_object* x_8; x_5 = lean_array_size(x_1); x_6 = 0; x_7 = lean_box(0); -x_8 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1(x_1, x_5, x_6, x_7, x_2, x_3, x_4); +x_8 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3(x_1, x_5, x_6, x_7, x_2, x_3, x_4); if (lean_obj_tag(x_8) == 0) { uint8_t x_9; @@ -2511,26 +2737,44 @@ return x_20; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___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_throwError___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___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___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__2(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___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_getConstInfo___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___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___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1(x_1, x_2, x_3, x_4); +x_5 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__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_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___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_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__2(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__2(x_1, x_2, x_3, x_4, x_5); lean_dec(x_2); return x_6; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___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) { _start: { size_t x_8; size_t x_9; lean_object* x_10; @@ -2538,7 +2782,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_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1(x_1, x_8, x_9, x_4, x_5, x_6, x_7); +x_10 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3(x_1, x_8, x_9, x_4, x_5, x_6, x_7); lean_dec(x_1); return x_10; } @@ -2564,7 +2808,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Deriving_TypeName__ _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__31; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__31; x_3 = l_Lean_Elab_initFn____x40_Lean_Elab_Deriving_TypeName___hyg_685____closed__1; x_4 = l_Lean_Elab_registerDerivingHandler(x_2, x_3, x_1); return x_4; @@ -2579,174 +2823,182 @@ _G_initialized = true; res = initialize_Lean_Elab_Deriving_Basic(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__1 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__1); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__2 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__2(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__2); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__3 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__3(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__3); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__4 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__4(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__4); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__5 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__5(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__5); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__6 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__6(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__6); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__7 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__7(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__7); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__8 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__8(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__8); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__9 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__9(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__9); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__10 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__10(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__10); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__11 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__11(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__11); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__12 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__12(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__12); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__13 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__13(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__13); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__14 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__14(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__14); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__15 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__15(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__15); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__16 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__16(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__16); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__17 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__17(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__17); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__18 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__18(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__18); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__19 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__19(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__19); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__20 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__20(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__20); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__21 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__21(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__21); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__22 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__22(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__22); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__23 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__23(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__23); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__24 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__24(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__24); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__25 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__25(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__25); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__26 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__26(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__26); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__27 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__27(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__27); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__28 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__28(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__28); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__29 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__29(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__29); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__30 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__30(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__30); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__31 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__31(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__31); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__32 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__32(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__32); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__33 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__33(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__33); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__34 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__34(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__34); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__35 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__35(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__35); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__36 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__36(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__36); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__37 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__37(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__37); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__38 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__38(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__38); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__39 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__39(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__39); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__40 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__40(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__40); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__41 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__41(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__41); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__42 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__42(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__42); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__43 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__43(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__43); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__44 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__44(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__44); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__45 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__45(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__45); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__46 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__46(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__46); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__47 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__47(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__47); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__48 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__48(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__48); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__49 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__49(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__49); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__50 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__50(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__50); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__51 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__51(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__51); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__52 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__52(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__52); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__53 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__53(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__53); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__54 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__54(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__54); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__55 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__55(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__55); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__56 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__56(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__56); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__57 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__57(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__57); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__58 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__58(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__58); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__59 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__59(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__59); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__60 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__60(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__60); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__61 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__61(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__61); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__62 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__62(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__62); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__63 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__63(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__63); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__64 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__64(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__64); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__65 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__65(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__65); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__66 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__66(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__66); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__67 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__67(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__67); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__68 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__68(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__68); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__69 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__69(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__69); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__70 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__70(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__70); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__71 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__71(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__71); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__72 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__72(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__72); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__73 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__73(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__73); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__74 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__74(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__74); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__75 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__75(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__75); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__76 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__76(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__76); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__77 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__77(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__77); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__78 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__78(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__78); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__79 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__79(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__1___closed__79); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__2___closed__1 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__2___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___lambda__2___closed__1); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__1 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__1); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__2 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__2(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__2); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__3 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__3(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__3); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__4 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__4(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__4); +l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__1 = _init_l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__1(); +lean_mark_persistent(l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__1); +l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__2 = _init_l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__2(); +lean_mark_persistent(l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__2); +l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__3 = _init_l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__3(); +lean_mark_persistent(l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__3); +l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__4 = _init_l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__4(); +lean_mark_persistent(l_Lean_getConstInfo___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__1___closed__4); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__1 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__1(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__1); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__2 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__2(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__2); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__3 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__3(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__3); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__4 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__4(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__4); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__5 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__5(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__5); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__6 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__6(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__6); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__7 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__7(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__7); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__8 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__8(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__8); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__9 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__9(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__9); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__10 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__10(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__10); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__11 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__11(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__11); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__12 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__12(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__12); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__13 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__13(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__13); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__14 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__14(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__14); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__15 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__15(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__15); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__16 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__16(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__16); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__17 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__17(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__17); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__18 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__18(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__18); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__19 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__19(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__19); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__20 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__20(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__20); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__21 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__21(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__21); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__22 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__22(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__22); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__23 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__23(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__23); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__24 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__24(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__24); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__25 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__25(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__25); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__26 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__26(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__26); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__27 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__27(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__27); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__28 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__28(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__28); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__29 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__29(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__29); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__30 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__30(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__30); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__31 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__31(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__31); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__32 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__32(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__32); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__33 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__33(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__33); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__34 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__34(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__34); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__35 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__35(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__35); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__36 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__36(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__36); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__37 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__37(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__37); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__38 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__38(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__38); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__39 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__39(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__39); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__40 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__40(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__40); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__41 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__41(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__41); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__42 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__42(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__42); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__43 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__43(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__43); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__44 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__44(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__44); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__45 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__45(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__45); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__46 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__46(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__46); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__47 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__47(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__47); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__48 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__48(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__48); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__49 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__49(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__49); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__50 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__50(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__50); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__51 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__51(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__51); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__52 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__52(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__52); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__53 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__53(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__53); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__54 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__54(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__54); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__55 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__55(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__55); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__56 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__56(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__56); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__57 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__57(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__57); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__58 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__58(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__58); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__59 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__59(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__59); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__60 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__60(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__60); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__61 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__61(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__61); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__62 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__62(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__62); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__63 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__63(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__63); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__64 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__64(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__64); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__65 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__65(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__65); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__66 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__66(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__66); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__67 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__67(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__67); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__68 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__68(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__68); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__69 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__69(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__69); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__70 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__70(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__70); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__71 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__71(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__71); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__72 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__72(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__72); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__73 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__73(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__73); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__74 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__74(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__74); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__75 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__75(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__75); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__76 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__76(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__76); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__77 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__77(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__77); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__78 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__78(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__78); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__79 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__79(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__1___closed__79); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__2___closed__1 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__2___closed__1(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___lambda__2___closed__1); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___closed__1 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___closed__1(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___closed__1); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___closed__2 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___closed__2(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___closed__2); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___closed__3 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___closed__3(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___closed__3); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___closed__4 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___closed__4(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Deriving_TypeName_0__Lean_Elab_deriveTypeNameInstance___spec__3___closed__4); l_Lean_Elab_initFn____x40_Lean_Elab_Deriving_TypeName___hyg_685____closed__1 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Deriving_TypeName___hyg_685____closed__1(); lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Deriving_TypeName___hyg_685____closed__1); res = l_Lean_Elab_initFn____x40_Lean_Elab_Deriving_TypeName___hyg_685_(lean_io_mk_world()); diff --git a/stage0/stdlib/Lean/Elab/Deriving/Util.c b/stage0/stdlib/Lean/Elab/Deriving/Util.c index ea5b18868001..15ae53e11f19 100644 --- a/stage0/stdlib/Lean/Elab/Deriving/Util.c +++ b/stage0/stdlib/Lean/Elab/Deriving/Util.c @@ -40,7 +40,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_mkContext___boxed(lean_object*, le static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_mkInstanceCmds___spec__1___lambda__1___closed__7; lean_object* lean_array_push(lean_object*, lean_object*); lean_object* l_Array_toSubarray___rarg(lean_object*, lean_object*, lean_object*); -uint8_t l_Array_contains___at_Lean_findField_x3f___spec__1(lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_mkInstanceCmds___spec__1___lambda__1___closed__13; LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_mkInstanceCmds(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -173,6 +172,7 @@ LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_mkContext___s static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_mkInstanceCmds___spec__1___lambda__1___closed__15; lean_object* l_Lean_Meta_forallBoundedTelescope___at_Lean_Elab_Term_addAutoBoundImplicits_x27___spec__2___rarg(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_mkLocalInstanceLetDecls___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_mkInstImplicitBinders___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at_Lean_Elab_Deriving_mkDiscrs___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -4097,7 +4097,7 @@ lean_inc(x_122); x_123 = lean_ctor_get(x_122, 0); lean_inc(x_123); lean_dec(x_122); -x_124 = l_Array_contains___at_Lean_findField_x3f___spec__1(x_3, x_123); +x_124 = l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(x_3, x_123); lean_dec(x_123); if (x_124 == 0) { diff --git a/stage0/stdlib/Lean/Elab/Frontend.c b/stage0/stdlib/Lean/Elab/Frontend.c index 72ec511f4ad8..9c01de8df868 100644 --- a/stage0/stdlib/Lean/Elab/Frontend.c +++ b/stage0/stdlib/Lean/Elab/Frontend.c @@ -16,7 +16,6 @@ extern "C" { lean_object* l_Lean_Language_Lean_process(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_profileit(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Frontend_processCommands___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_runFrontend___spec__2(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Frontend_setMessages___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Firefox_Profile_export(lean_object*, double, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Json_compress(lean_object*); @@ -53,7 +52,6 @@ lean_object* l_Lean_Language_SnapshotTree_getAll(lean_object*); lean_object* l_Lean_Exception_toMessageData(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Frontend_runCommandElabM(lean_object*); static double l_Lean_Elab_runFrontend___closed__1; -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_runFrontend___spec__1(lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Elab_Frontend_getCommandState___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_runFrontend___lambda__3___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_runFrontend___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -64,30 +62,33 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Frontend_getCommandState___boxed(lean_objec size_t lean_usize_of_nat(lean_object*); uint8_t l_Lean_Parser_isTerminalCommand(lean_object*); lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonProfile____x40_Lean_Util_Profiler___hyg_3680_(lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_runFrontend___spec__3___boxed(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_Frontend_elabCommandAtFrontend(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Language_Lean_processCommands(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Option_setIfNotSet___at_Lean_Elab_runFrontend___spec__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_runFrontend___closed__3; -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_runFrontend___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_filterMapM___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__3___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__2(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Frontend_runCommandElabM___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__6(lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Elab_process___closed__2; LEAN_EXPORT lean_object* l_Array_filterMapM___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__3___boxed(lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Frontend_setParserState___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_mkInputContext(lean_object*, lean_object*, uint8_t); lean_object* lean_st_mk_ref(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__5(lean_object*, size_t, size_t, lean_object*); lean_object* l_Array_toPArray_x27___rarg(lean_object*); static lean_object* l_Lean_Elab_runFrontend___closed__4; lean_object* lean_io_mono_nanos_now(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Frontend_elabCommandAtFrontend___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Option_set___at_Lean_Elab_Term_withoutMacroStackAtErr___spec__1(lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Elab_Frontend_processCommand___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__5(size_t, size_t, lean_object*); extern lean_object* l_Lean_Language_Lean_internal_cmdlineSnapshots; lean_object* lean_task_get_own(lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Option_setIfNotSet___at_Lean_Elab_runFrontend___spec__1(lean_object*, lean_object*, uint8_t); lean_object* l_Lean_Server_ModuleRefs_toLspModuleRefs(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__1; double l_Float_ofScientific(lean_object*, uint8_t, lean_object*); @@ -95,17 +96,19 @@ static lean_object* l_Lean_Elab_Frontend_runCommandElabM___rarg___closed__2; LEAN_EXPORT lean_object* lean_run_frontend(lean_object*, lean_object*, lean_object*, lean_object*, uint32_t, lean_object*, uint8_t, lean_object*); lean_object* l___private_Lean_Server_References_0__Lean_Server_toJsonIlean____x40_Lean_Server_References___hyg_1478_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Frontend_setMessages(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_runFrontend___spec__1___boxed(lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_NameSet_empty; LEAN_EXPORT uint8_t l_Lean_Elab_runFrontend___lambda__3(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Frontend_getCommandState(lean_object*); +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_runFrontend___spec__2(lean_object*, size_t, size_t); static lean_object* l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__3; uint8_t lean_nat_dec_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Frontend_getInputContext(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_IO_processCommands(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_runFrontend___spec__2___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Language_Lean_instToSnapshotTreeCommandParsedSnapshot_go(lean_object*); lean_object* l_Lean_Language_Lean_waitForFinalCmdState_x3f(lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_runFrontend___spec__3(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_IO_processCommandsIncrementally_go(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Frontend_processCommand___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Option_get_x3f___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessages___spec__1(lean_object*, lean_object*); @@ -113,6 +116,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_runFrontend___lambda__1(lean_object*, lean_ static lean_object* l_Lean_Elab_runFrontend___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Frontend_processCommand(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__4(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__5___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_runFrontend___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_firstFrontendMacroScope; extern lean_object* l_Lean_Elab_Command_instInhabitedScope; @@ -121,6 +125,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Frontend_setCommandState(lean_object*, lean LEAN_EXPORT lean_object* l_Lean_Elab_process(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Frontend_updateCmdPos___rarg(lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Language_SnapshotTask_map___rarg(lean_object*, lean_object*, lean_object*, uint8_t); lean_object* l_Lean_MessageLog_append(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_runFrontend___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, double, lean_object*, lean_object*); @@ -136,11 +141,11 @@ extern lean_object* l_Lean_trace_profiler_output; lean_object* lean_array_get_size(lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Frontend_setParserState(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); lean_object* lean_mk_empty_environment(uint32_t, lean_object*); static lean_object* l_Lean_Elab_Frontend_processCommand___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Frontend_getParserState___boxed(lean_object*); +uint8_t l_Lean_KVMap_contains(lean_object*, lean_object*); lean_object* l_Lean_Parser_parseCommand(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_runFrontend___lambda__5(lean_object*, lean_object*, lean_object*); lean_object* lean_array_uset(lean_object*, size_t, lean_object*); @@ -2063,18 +2068,25 @@ return x_3; } else { -lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; size_t x_9; size_t x_10; lean_object* x_11; +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; size_t x_12; size_t x_13; lean_object* x_14; x_5 = lean_array_uget(x_3, x_2); x_6 = lean_unsigned_to_nat(0u); x_7 = lean_array_uset(x_3, x_2, x_6); -x_8 = lean_ctor_get(x_5, 2); +x_8 = lean_ctor_get(x_5, 4); lean_inc(x_8); lean_dec(x_5); -x_9 = 1; -x_10 = lean_usize_add(x_2, x_9); -x_11 = lean_array_uset(x_7, x_2, x_8); -x_2 = x_10; -x_3 = x_11; +x_9 = l_Lean_Language_SnapshotTask_get___rarg(x_8); +x_10 = lean_ctor_get(x_9, 0); +lean_inc(x_10); +lean_dec(x_9); +x_11 = lean_ctor_get(x_10, 2); +lean_inc(x_11); +lean_dec(x_10); +x_12 = 1; +x_13 = lean_usize_add(x_2, x_12); +x_14 = lean_array_uset(x_7, x_2, x_11); +x_2 = x_13; +x_3 = x_14; goto _start; } } @@ -2157,7 +2169,34 @@ return x_12; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__5(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__5(size_t x_1, size_t x_2, lean_object* x_3) { +_start: +{ +uint8_t x_4; +x_4 = lean_usize_dec_lt(x_2, x_1); +if (x_4 == 0) +{ +return x_3; +} +else +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; size_t x_9; size_t x_10; lean_object* x_11; +x_5 = lean_array_uget(x_3, x_2); +x_6 = lean_unsigned_to_nat(0u); +x_7 = lean_array_uset(x_3, x_2, x_6); +x_8 = lean_ctor_get(x_5, 1); +lean_inc(x_8); +lean_dec(x_5); +x_9 = 1; +x_10 = lean_usize_add(x_2, x_9); +x_11 = lean_array_uset(x_7, x_2, x_8); +x_2 = x_10; +x_3 = x_11; +goto _start; +} +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__6(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { uint8_t x_5; @@ -2187,28 +2226,28 @@ x_6 = lean_task_get_own(x_3); x_7 = !lean_is_exclusive(x_6); if (x_7 == 0) { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +lean_object* x_8; lean_object* x_9; lean_object* x_10; x_8 = lean_ctor_get(x_6, 0); x_9 = lean_ctor_get(x_6, 1); -x_10 = lean_ctor_get(x_8, 1); -lean_inc(x_10); -x_11 = lean_array_push(x_4, x_10); +lean_inc(x_8); +x_10 = lean_array_push(x_4, x_8); if (lean_obj_tag(x_9) == 0) { -lean_object* x_12; lean_object* x_13; size_t x_14; size_t x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; +lean_object* x_11; lean_object* x_12; size_t x_13; size_t x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; size_t x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; lean_inc(x_2); -x_12 = l_Lean_Language_Lean_instToSnapshotTreeCommandParsedSnapshot_go(x_2); -x_13 = l_Lean_Language_SnapshotTree_getAll(x_12); -x_14 = lean_array_size(x_13); -x_15 = 0; -lean_inc(x_13); -x_16 = l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__1(x_14, x_15, x_13); -x_17 = lean_array_get_size(x_16); -x_18 = lean_unsigned_to_nat(0u); -x_19 = lean_nat_dec_lt(x_18, x_17); -x_20 = l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__2(x_14, x_15, x_13); +x_11 = l_Lean_Language_Lean_instToSnapshotTreeCommandParsedSnapshot_go(x_2); +x_12 = l_Lean_Language_SnapshotTree_getAll(x_11); +x_13 = lean_array_size(x_12); +x_14 = 0; +x_15 = l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__1(x_13, x_14, x_12); +x_16 = lean_array_get_size(x_15); +x_17 = lean_unsigned_to_nat(0u); +x_18 = lean_nat_dec_lt(x_17, x_16); +x_19 = lean_array_size(x_10); +lean_inc(x_10); +x_20 = l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__2(x_19, x_14, x_10); x_21 = lean_array_get_size(x_20); -x_22 = l_Array_filterMapM___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__3(x_20, x_18, x_21); +x_22 = l_Array_filterMapM___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__3(x_20, x_17, x_21); lean_dec(x_21); lean_dec(x_20); x_23 = l_Array_toPArray_x27___rarg(x_22); @@ -2229,117 +2268,114 @@ lean_dec(x_29); x_30 = !lean_is_exclusive(x_28); if (x_30 == 0) { -lean_object* x_31; +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; x_31 = lean_ctor_get(x_28, 1); lean_dec(x_31); lean_ctor_set(x_28, 1, x_23); -if (x_19 == 0) -{ -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; -lean_dec(x_17); -lean_dec(x_16); x_32 = lean_ctor_get(x_8, 2); lean_inc(x_32); lean_dec(x_8); x_33 = lean_ctor_get(x_32, 0); lean_inc(x_33); -x_34 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; -lean_ctor_set(x_26, 1, x_34); -x_35 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_35, 0, x_26); -lean_ctor_set(x_35, 1, x_32); -lean_ctor_set(x_35, 2, x_33); -lean_ctor_set(x_35, 3, x_11); -x_36 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_36, 0, x_35); -lean_ctor_set(x_36, 1, x_1); -lean_ctor_set(x_36, 2, x_2); +x_34 = l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__5(x_19, x_14, x_10); +if (x_18 == 0) +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; +lean_dec(x_16); +lean_dec(x_15); +x_35 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; +lean_ctor_set(x_26, 1, x_35); +x_36 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_36, 0, x_26); +lean_ctor_set(x_36, 1, x_32); +lean_ctor_set(x_36, 2, x_33); +lean_ctor_set(x_36, 3, x_34); +x_37 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_37, 0, x_36); +lean_ctor_set(x_37, 1, x_1); +lean_ctor_set(x_37, 2, x_2); lean_ctor_set(x_6, 1, x_5); -lean_ctor_set(x_6, 0, x_36); +lean_ctor_set(x_6, 0, x_37); return x_6; } else { -lean_object* x_37; lean_object* x_38; uint8_t x_39; -x_37 = lean_ctor_get(x_8, 2); -lean_inc(x_37); -lean_dec(x_8); -x_38 = lean_ctor_get(x_37, 0); -lean_inc(x_38); -x_39 = lean_nat_dec_le(x_17, x_17); -if (x_39 == 0) +uint8_t x_38; +x_38 = lean_nat_dec_le(x_16, x_16); +if (x_38 == 0) { -lean_object* x_40; lean_object* x_41; lean_object* x_42; -lean_dec(x_17); +lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_dec(x_16); -x_40 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; -lean_ctor_set(x_26, 1, x_40); -x_41 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_41, 0, x_26); -lean_ctor_set(x_41, 1, x_37); -lean_ctor_set(x_41, 2, x_38); -lean_ctor_set(x_41, 3, x_11); -x_42 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_42, 0, x_41); -lean_ctor_set(x_42, 1, x_1); -lean_ctor_set(x_42, 2, x_2); +lean_dec(x_15); +x_39 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; +lean_ctor_set(x_26, 1, x_39); +x_40 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_40, 0, x_26); +lean_ctor_set(x_40, 1, x_32); +lean_ctor_set(x_40, 2, x_33); +lean_ctor_set(x_40, 3, x_34); +x_41 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_41, 0, x_40); +lean_ctor_set(x_41, 1, x_1); +lean_ctor_set(x_41, 2, x_2); lean_ctor_set(x_6, 1, x_5); -lean_ctor_set(x_6, 0, x_42); +lean_ctor_set(x_6, 0, x_41); return x_6; } else { -size_t x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_43 = lean_usize_of_nat(x_17); -lean_dec(x_17); -x_44 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; -x_45 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__5(x_16, x_15, x_43, x_44); +size_t x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_42 = lean_usize_of_nat(x_16); lean_dec(x_16); -lean_ctor_set(x_26, 1, x_45); -x_46 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_46, 0, x_26); -lean_ctor_set(x_46, 1, x_37); -lean_ctor_set(x_46, 2, x_38); -lean_ctor_set(x_46, 3, x_11); -x_47 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_47, 0, x_46); -lean_ctor_set(x_47, 1, x_1); -lean_ctor_set(x_47, 2, x_2); +x_43 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; +x_44 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__6(x_15, x_14, x_42, x_43); +lean_dec(x_15); +lean_ctor_set(x_26, 1, x_44); +x_45 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_45, 0, x_26); +lean_ctor_set(x_45, 1, x_32); +lean_ctor_set(x_45, 2, x_33); +lean_ctor_set(x_45, 3, x_34); +x_46 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_46, 0, x_45); +lean_ctor_set(x_46, 1, x_1); +lean_ctor_set(x_46, 2, x_2); lean_ctor_set(x_6, 1, x_5); -lean_ctor_set(x_6, 0, x_47); +lean_ctor_set(x_6, 0, x_46); return x_6; } } } else { -uint8_t x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_ctor_get_uint8(x_28, sizeof(void*)*2); -x_49 = lean_ctor_get(x_28, 0); -lean_inc(x_49); +uint8_t x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_47 = lean_ctor_get_uint8(x_28, sizeof(void*)*2); +x_48 = lean_ctor_get(x_28, 0); +lean_inc(x_48); lean_dec(x_28); -x_50 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_50, 0, x_49); -lean_ctor_set(x_50, 1, x_23); -lean_ctor_set_uint8(x_50, sizeof(void*)*2, x_48); -if (x_19 == 0) +x_49 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_49, 0, x_48); +lean_ctor_set(x_49, 1, x_23); +lean_ctor_set_uint8(x_49, sizeof(void*)*2, x_47); +x_50 = lean_ctor_get(x_8, 2); +lean_inc(x_50); +lean_dec(x_8); +x_51 = lean_ctor_get(x_50, 0); +lean_inc(x_51); +x_52 = l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__5(x_19, x_14, x_10); +if (x_18 == 0) { -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; -lean_dec(x_17); +lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_dec(x_16); -x_51 = lean_ctor_get(x_8, 2); -lean_inc(x_51); -lean_dec(x_8); -x_52 = lean_ctor_get(x_51, 0); -lean_inc(x_52); +lean_dec(x_15); x_53 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; -lean_ctor_set(x_26, 6, x_50); +lean_ctor_set(x_26, 6, x_49); lean_ctor_set(x_26, 1, x_53); x_54 = lean_alloc_ctor(0, 4, 0); lean_ctor_set(x_54, 0, x_26); -lean_ctor_set(x_54, 1, x_51); -lean_ctor_set(x_54, 2, x_52); -lean_ctor_set(x_54, 3, x_11); +lean_ctor_set(x_54, 1, x_50); +lean_ctor_set(x_54, 2, x_51); +lean_ctor_set(x_54, 3, x_52); x_55 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_55, 0, x_54); lean_ctor_set(x_55, 1, x_1); @@ -2350,55 +2386,50 @@ return x_6; } else { -lean_object* x_56; lean_object* x_57; uint8_t x_58; -x_56 = lean_ctor_get(x_8, 2); -lean_inc(x_56); -lean_dec(x_8); -x_57 = lean_ctor_get(x_56, 0); -lean_inc(x_57); -x_58 = lean_nat_dec_le(x_17, x_17); -if (x_58 == 0) +uint8_t x_56; +x_56 = lean_nat_dec_le(x_16, x_16); +if (x_56 == 0) { -lean_object* x_59; lean_object* x_60; lean_object* x_61; -lean_dec(x_17); +lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_dec(x_16); -x_59 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; -lean_ctor_set(x_26, 6, x_50); -lean_ctor_set(x_26, 1, x_59); -x_60 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_60, 0, x_26); -lean_ctor_set(x_60, 1, x_56); -lean_ctor_set(x_60, 2, x_57); -lean_ctor_set(x_60, 3, x_11); -x_61 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_61, 0, x_60); -lean_ctor_set(x_61, 1, x_1); -lean_ctor_set(x_61, 2, x_2); +lean_dec(x_15); +x_57 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; +lean_ctor_set(x_26, 6, x_49); +lean_ctor_set(x_26, 1, x_57); +x_58 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_58, 0, x_26); +lean_ctor_set(x_58, 1, x_50); +lean_ctor_set(x_58, 2, x_51); +lean_ctor_set(x_58, 3, x_52); +x_59 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_59, 0, x_58); +lean_ctor_set(x_59, 1, x_1); +lean_ctor_set(x_59, 2, x_2); lean_ctor_set(x_6, 1, x_5); -lean_ctor_set(x_6, 0, x_61); +lean_ctor_set(x_6, 0, x_59); return x_6; } else { -size_t x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_62 = lean_usize_of_nat(x_17); -lean_dec(x_17); -x_63 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; -x_64 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__5(x_16, x_15, x_62, x_63); +size_t x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; +x_60 = lean_usize_of_nat(x_16); lean_dec(x_16); -lean_ctor_set(x_26, 6, x_50); -lean_ctor_set(x_26, 1, x_64); -x_65 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_65, 0, x_26); -lean_ctor_set(x_65, 1, x_56); -lean_ctor_set(x_65, 2, x_57); -lean_ctor_set(x_65, 3, x_11); -x_66 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_66, 0, x_65); -lean_ctor_set(x_66, 1, x_1); -lean_ctor_set(x_66, 2, x_2); +x_61 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; +x_62 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__6(x_15, x_14, x_60, x_61); +lean_dec(x_15); +lean_ctor_set(x_26, 6, x_49); +lean_ctor_set(x_26, 1, x_62); +x_63 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_63, 0, x_26); +lean_ctor_set(x_63, 1, x_50); +lean_ctor_set(x_63, 2, x_51); +lean_ctor_set(x_63, 3, x_52); +x_64 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_64, 0, x_63); +lean_ctor_set(x_64, 1, x_1); +lean_ctor_set(x_64, 2, x_2); lean_ctor_set(x_6, 1, x_5); -lean_ctor_set(x_6, 0, x_66); +lean_ctor_set(x_6, 0, x_64); return x_6; } } @@ -2406,139 +2437,135 @@ return x_6; } else { -lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; uint8_t x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_67 = lean_ctor_get(x_26, 6); -x_68 = lean_ctor_get(x_26, 0); -x_69 = lean_ctor_get(x_26, 2); -x_70 = lean_ctor_get(x_26, 3); -x_71 = lean_ctor_get(x_26, 4); -x_72 = lean_ctor_get(x_26, 5); -x_73 = lean_ctor_get(x_26, 7); -lean_inc(x_73); -lean_inc(x_67); -lean_inc(x_72); +lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; uint8_t x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; +x_65 = lean_ctor_get(x_26, 6); +x_66 = lean_ctor_get(x_26, 0); +x_67 = lean_ctor_get(x_26, 2); +x_68 = lean_ctor_get(x_26, 3); +x_69 = lean_ctor_get(x_26, 4); +x_70 = lean_ctor_get(x_26, 5); +x_71 = lean_ctor_get(x_26, 7); lean_inc(x_71); +lean_inc(x_65); lean_inc(x_70); lean_inc(x_69); lean_inc(x_68); +lean_inc(x_67); +lean_inc(x_66); lean_dec(x_26); -x_74 = lean_ctor_get_uint8(x_67, sizeof(void*)*2); -x_75 = lean_ctor_get(x_67, 0); -lean_inc(x_75); -if (lean_is_exclusive(x_67)) { - lean_ctor_release(x_67, 0); - lean_ctor_release(x_67, 1); - x_76 = x_67; +x_72 = lean_ctor_get_uint8(x_65, sizeof(void*)*2); +x_73 = lean_ctor_get(x_65, 0); +lean_inc(x_73); +if (lean_is_exclusive(x_65)) { + lean_ctor_release(x_65, 0); + lean_ctor_release(x_65, 1); + x_74 = x_65; } else { - lean_dec_ref(x_67); - x_76 = lean_box(0); + lean_dec_ref(x_65); + x_74 = lean_box(0); } -if (lean_is_scalar(x_76)) { - x_77 = lean_alloc_ctor(0, 2, 1); +if (lean_is_scalar(x_74)) { + x_75 = lean_alloc_ctor(0, 2, 1); } else { - x_77 = x_76; + x_75 = x_74; } -lean_ctor_set(x_77, 0, x_75); -lean_ctor_set(x_77, 1, x_23); -lean_ctor_set_uint8(x_77, sizeof(void*)*2, x_74); -if (x_19 == 0) +lean_ctor_set(x_75, 0, x_73); +lean_ctor_set(x_75, 1, x_23); +lean_ctor_set_uint8(x_75, sizeof(void*)*2, x_72); +x_76 = lean_ctor_get(x_8, 2); +lean_inc(x_76); +lean_dec(x_8); +x_77 = lean_ctor_get(x_76, 0); +lean_inc(x_77); +x_78 = l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__5(x_19, x_14, x_10); +if (x_18 == 0) { -lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; -lean_dec(x_17); +lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_dec(x_16); -x_78 = lean_ctor_get(x_8, 2); -lean_inc(x_78); -lean_dec(x_8); -x_79 = lean_ctor_get(x_78, 0); -lean_inc(x_79); -x_80 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; -x_81 = lean_alloc_ctor(0, 8, 0); -lean_ctor_set(x_81, 0, x_68); -lean_ctor_set(x_81, 1, x_80); -lean_ctor_set(x_81, 2, x_69); -lean_ctor_set(x_81, 3, x_70); -lean_ctor_set(x_81, 4, x_71); -lean_ctor_set(x_81, 5, x_72); -lean_ctor_set(x_81, 6, x_77); -lean_ctor_set(x_81, 7, x_73); -x_82 = lean_alloc_ctor(0, 4, 0); +lean_dec(x_15); +x_79 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; +x_80 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_80, 0, x_66); +lean_ctor_set(x_80, 1, x_79); +lean_ctor_set(x_80, 2, x_67); +lean_ctor_set(x_80, 3, x_68); +lean_ctor_set(x_80, 4, x_69); +lean_ctor_set(x_80, 5, x_70); +lean_ctor_set(x_80, 6, x_75); +lean_ctor_set(x_80, 7, x_71); +x_81 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_81, 0, x_80); +lean_ctor_set(x_81, 1, x_76); +lean_ctor_set(x_81, 2, x_77); +lean_ctor_set(x_81, 3, x_78); +x_82 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_82, 0, x_81); -lean_ctor_set(x_82, 1, x_78); -lean_ctor_set(x_82, 2, x_79); -lean_ctor_set(x_82, 3, x_11); -x_83 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_83, 0, x_82); -lean_ctor_set(x_83, 1, x_1); -lean_ctor_set(x_83, 2, x_2); +lean_ctor_set(x_82, 1, x_1); +lean_ctor_set(x_82, 2, x_2); lean_ctor_set(x_6, 1, x_5); -lean_ctor_set(x_6, 0, x_83); +lean_ctor_set(x_6, 0, x_82); return x_6; } else { -lean_object* x_84; lean_object* x_85; uint8_t x_86; -x_84 = lean_ctor_get(x_8, 2); -lean_inc(x_84); -lean_dec(x_8); -x_85 = lean_ctor_get(x_84, 0); -lean_inc(x_85); -x_86 = lean_nat_dec_le(x_17, x_17); -if (x_86 == 0) +uint8_t x_83; +x_83 = lean_nat_dec_le(x_16, x_16); +if (x_83 == 0) { -lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; -lean_dec(x_17); +lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_dec(x_16); -x_87 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; -x_88 = lean_alloc_ctor(0, 8, 0); -lean_ctor_set(x_88, 0, x_68); -lean_ctor_set(x_88, 1, x_87); -lean_ctor_set(x_88, 2, x_69); -lean_ctor_set(x_88, 3, x_70); -lean_ctor_set(x_88, 4, x_71); -lean_ctor_set(x_88, 5, x_72); -lean_ctor_set(x_88, 6, x_77); -lean_ctor_set(x_88, 7, x_73); -x_89 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_89, 0, x_88); -lean_ctor_set(x_89, 1, x_84); -lean_ctor_set(x_89, 2, x_85); -lean_ctor_set(x_89, 3, x_11); -x_90 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_90, 0, x_89); -lean_ctor_set(x_90, 1, x_1); -lean_ctor_set(x_90, 2, x_2); +lean_dec(x_15); +x_84 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; +x_85 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_85, 0, x_66); +lean_ctor_set(x_85, 1, x_84); +lean_ctor_set(x_85, 2, x_67); +lean_ctor_set(x_85, 3, x_68); +lean_ctor_set(x_85, 4, x_69); +lean_ctor_set(x_85, 5, x_70); +lean_ctor_set(x_85, 6, x_75); +lean_ctor_set(x_85, 7, x_71); +x_86 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_86, 0, x_85); +lean_ctor_set(x_86, 1, x_76); +lean_ctor_set(x_86, 2, x_77); +lean_ctor_set(x_86, 3, x_78); +x_87 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_87, 0, x_86); +lean_ctor_set(x_87, 1, x_1); +lean_ctor_set(x_87, 2, x_2); lean_ctor_set(x_6, 1, x_5); -lean_ctor_set(x_6, 0, x_90); +lean_ctor_set(x_6, 0, x_87); return x_6; } else { -size_t x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; -x_91 = lean_usize_of_nat(x_17); -lean_dec(x_17); -x_92 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; -x_93 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__5(x_16, x_15, x_91, x_92); +size_t x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; +x_88 = lean_usize_of_nat(x_16); lean_dec(x_16); -x_94 = lean_alloc_ctor(0, 8, 0); -lean_ctor_set(x_94, 0, x_68); -lean_ctor_set(x_94, 1, x_93); -lean_ctor_set(x_94, 2, x_69); -lean_ctor_set(x_94, 3, x_70); -lean_ctor_set(x_94, 4, x_71); -lean_ctor_set(x_94, 5, x_72); -lean_ctor_set(x_94, 6, x_77); -lean_ctor_set(x_94, 7, x_73); -x_95 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_95, 0, x_94); -lean_ctor_set(x_95, 1, x_84); -lean_ctor_set(x_95, 2, x_85); -lean_ctor_set(x_95, 3, x_11); -x_96 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_96, 0, x_95); -lean_ctor_set(x_96, 1, x_1); -lean_ctor_set(x_96, 2, x_2); +x_89 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; +x_90 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__6(x_15, x_14, x_88, x_89); +lean_dec(x_15); +x_91 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_91, 0, x_66); +lean_ctor_set(x_91, 1, x_90); +lean_ctor_set(x_91, 2, x_67); +lean_ctor_set(x_91, 3, x_68); +lean_ctor_set(x_91, 4, x_69); +lean_ctor_set(x_91, 5, x_70); +lean_ctor_set(x_91, 6, x_75); +lean_ctor_set(x_91, 7, x_71); +x_92 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_92, 0, x_91); +lean_ctor_set(x_92, 1, x_76); +lean_ctor_set(x_92, 2, x_77); +lean_ctor_set(x_92, 3, x_78); +x_93 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_93, 0, x_92); +lean_ctor_set(x_93, 1, x_1); +lean_ctor_set(x_93, 2, x_2); lean_ctor_set(x_6, 1, x_5); -lean_ctor_set(x_6, 0, x_96); +lean_ctor_set(x_6, 0, x_93); return x_6; } } @@ -2546,233 +2573,229 @@ return x_6; } else { -lean_object* x_97; lean_object* x_98; +lean_object* x_94; lean_object* x_95; lean_free_object(x_6); lean_dec(x_8); -x_97 = lean_ctor_get(x_9, 0); -lean_inc(x_97); +x_94 = lean_ctor_get(x_9, 0); +lean_inc(x_94); lean_dec(x_9); -x_98 = lean_ctor_get(x_97, 1); -lean_inc(x_98); -lean_dec(x_97); -x_3 = x_98; -x_4 = x_11; +x_95 = lean_ctor_get(x_94, 1); +lean_inc(x_95); +lean_dec(x_94); +x_3 = x_95; +x_4 = x_10; goto _start; } } else { -lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; -x_100 = lean_ctor_get(x_6, 0); -x_101 = lean_ctor_get(x_6, 1); -lean_inc(x_101); -lean_inc(x_100); +lean_object* x_97; lean_object* x_98; lean_object* x_99; +x_97 = lean_ctor_get(x_6, 0); +x_98 = lean_ctor_get(x_6, 1); +lean_inc(x_98); +lean_inc(x_97); lean_dec(x_6); -x_102 = lean_ctor_get(x_100, 1); -lean_inc(x_102); -x_103 = lean_array_push(x_4, x_102); -if (lean_obj_tag(x_101) == 0) +lean_inc(x_97); +x_99 = lean_array_push(x_4, x_97); +if (lean_obj_tag(x_98) == 0) { -lean_object* x_104; lean_object* x_105; size_t x_106; size_t x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; uint8_t x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; uint8_t x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; +lean_object* x_100; lean_object* x_101; size_t x_102; size_t x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; uint8_t x_107; size_t x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; uint8_t x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_inc(x_2); -x_104 = l_Lean_Language_Lean_instToSnapshotTreeCommandParsedSnapshot_go(x_2); -x_105 = l_Lean_Language_SnapshotTree_getAll(x_104); -x_106 = lean_array_size(x_105); -x_107 = 0; -lean_inc(x_105); -x_108 = l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__1(x_106, x_107, x_105); -x_109 = lean_array_get_size(x_108); -x_110 = lean_unsigned_to_nat(0u); -x_111 = lean_nat_dec_lt(x_110, x_109); -x_112 = l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__2(x_106, x_107, x_105); -x_113 = lean_array_get_size(x_112); -x_114 = l_Array_filterMapM___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__3(x_112, x_110, x_113); -lean_dec(x_113); -lean_dec(x_112); -x_115 = l_Array_toPArray_x27___rarg(x_114); +x_100 = l_Lean_Language_Lean_instToSnapshotTreeCommandParsedSnapshot_go(x_2); +x_101 = l_Lean_Language_SnapshotTree_getAll(x_100); +x_102 = lean_array_size(x_101); +x_103 = 0; +x_104 = l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__1(x_102, x_103, x_101); +x_105 = lean_array_get_size(x_104); +x_106 = lean_unsigned_to_nat(0u); +x_107 = lean_nat_dec_lt(x_106, x_105); +x_108 = lean_array_size(x_99); +lean_inc(x_99); +x_109 = l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__2(x_108, x_103, x_99); +x_110 = lean_array_get_size(x_109); +x_111 = l_Array_filterMapM___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__3(x_109, x_106, x_110); +lean_dec(x_110); +lean_dec(x_109); +x_112 = l_Array_toPArray_x27___rarg(x_111); +lean_dec(x_111); +x_113 = lean_ctor_get(x_97, 4); +lean_inc(x_113); +x_114 = l_Lean_Language_SnapshotTask_get___rarg(x_113); +x_115 = lean_ctor_get(x_114, 1); +lean_inc(x_115); lean_dec(x_114); -x_116 = lean_ctor_get(x_100, 4); +x_116 = lean_ctor_get(x_115, 6); lean_inc(x_116); -x_117 = l_Lean_Language_SnapshotTask_get___rarg(x_116); -x_118 = lean_ctor_get(x_117, 1); +x_117 = lean_ctor_get(x_115, 0); +lean_inc(x_117); +x_118 = lean_ctor_get(x_115, 2); lean_inc(x_118); -lean_dec(x_117); -x_119 = lean_ctor_get(x_118, 6); +x_119 = lean_ctor_get(x_115, 3); lean_inc(x_119); -x_120 = lean_ctor_get(x_118, 0); +x_120 = lean_ctor_get(x_115, 4); lean_inc(x_120); -x_121 = lean_ctor_get(x_118, 2); +x_121 = lean_ctor_get(x_115, 5); lean_inc(x_121); -x_122 = lean_ctor_get(x_118, 3); +x_122 = lean_ctor_get(x_115, 7); lean_inc(x_122); -x_123 = lean_ctor_get(x_118, 4); -lean_inc(x_123); -x_124 = lean_ctor_get(x_118, 5); -lean_inc(x_124); -x_125 = lean_ctor_get(x_118, 7); -lean_inc(x_125); -if (lean_is_exclusive(x_118)) { - lean_ctor_release(x_118, 0); - lean_ctor_release(x_118, 1); - lean_ctor_release(x_118, 2); - lean_ctor_release(x_118, 3); - lean_ctor_release(x_118, 4); - lean_ctor_release(x_118, 5); - lean_ctor_release(x_118, 6); - lean_ctor_release(x_118, 7); - x_126 = x_118; +if (lean_is_exclusive(x_115)) { + lean_ctor_release(x_115, 0); + lean_ctor_release(x_115, 1); + lean_ctor_release(x_115, 2); + lean_ctor_release(x_115, 3); + lean_ctor_release(x_115, 4); + lean_ctor_release(x_115, 5); + lean_ctor_release(x_115, 6); + lean_ctor_release(x_115, 7); + x_123 = x_115; } else { - lean_dec_ref(x_118); - x_126 = lean_box(0); + lean_dec_ref(x_115); + x_123 = lean_box(0); } -x_127 = lean_ctor_get_uint8(x_119, sizeof(void*)*2); -x_128 = lean_ctor_get(x_119, 0); -lean_inc(x_128); -if (lean_is_exclusive(x_119)) { - lean_ctor_release(x_119, 0); - lean_ctor_release(x_119, 1); - x_129 = x_119; +x_124 = lean_ctor_get_uint8(x_116, sizeof(void*)*2); +x_125 = lean_ctor_get(x_116, 0); +lean_inc(x_125); +if (lean_is_exclusive(x_116)) { + lean_ctor_release(x_116, 0); + lean_ctor_release(x_116, 1); + x_126 = x_116; } else { - lean_dec_ref(x_119); - x_129 = lean_box(0); + lean_dec_ref(x_116); + x_126 = lean_box(0); } -if (lean_is_scalar(x_129)) { - x_130 = lean_alloc_ctor(0, 2, 1); +if (lean_is_scalar(x_126)) { + x_127 = lean_alloc_ctor(0, 2, 1); } else { - x_130 = x_129; + x_127 = x_126; } -lean_ctor_set(x_130, 0, x_128); -lean_ctor_set(x_130, 1, x_115); -lean_ctor_set_uint8(x_130, sizeof(void*)*2, x_127); -if (x_111 == 0) +lean_ctor_set(x_127, 0, x_125); +lean_ctor_set(x_127, 1, x_112); +lean_ctor_set_uint8(x_127, sizeof(void*)*2, x_124); +x_128 = lean_ctor_get(x_97, 2); +lean_inc(x_128); +lean_dec(x_97); +x_129 = lean_ctor_get(x_128, 0); +lean_inc(x_129); +x_130 = l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__5(x_108, x_103, x_99); +if (x_107 == 0) { -lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; -lean_dec(x_109); -lean_dec(x_108); -x_131 = lean_ctor_get(x_100, 2); -lean_inc(x_131); -lean_dec(x_100); -x_132 = lean_ctor_get(x_131, 0); -lean_inc(x_132); -x_133 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; -if (lean_is_scalar(x_126)) { - x_134 = lean_alloc_ctor(0, 8, 0); +lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; +lean_dec(x_105); +lean_dec(x_104); +x_131 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; +if (lean_is_scalar(x_123)) { + x_132 = lean_alloc_ctor(0, 8, 0); } else { - x_134 = x_126; -} -lean_ctor_set(x_134, 0, x_120); -lean_ctor_set(x_134, 1, x_133); -lean_ctor_set(x_134, 2, x_121); -lean_ctor_set(x_134, 3, x_122); -lean_ctor_set(x_134, 4, x_123); -lean_ctor_set(x_134, 5, x_124); -lean_ctor_set(x_134, 6, x_130); -lean_ctor_set(x_134, 7, x_125); -x_135 = lean_alloc_ctor(0, 4, 0); + x_132 = x_123; +} +lean_ctor_set(x_132, 0, x_117); +lean_ctor_set(x_132, 1, x_131); +lean_ctor_set(x_132, 2, x_118); +lean_ctor_set(x_132, 3, x_119); +lean_ctor_set(x_132, 4, x_120); +lean_ctor_set(x_132, 5, x_121); +lean_ctor_set(x_132, 6, x_127); +lean_ctor_set(x_132, 7, x_122); +x_133 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_133, 0, x_132); +lean_ctor_set(x_133, 1, x_128); +lean_ctor_set(x_133, 2, x_129); +lean_ctor_set(x_133, 3, x_130); +x_134 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_134, 0, x_133); +lean_ctor_set(x_134, 1, x_1); +lean_ctor_set(x_134, 2, x_2); +x_135 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_135, 0, x_134); -lean_ctor_set(x_135, 1, x_131); -lean_ctor_set(x_135, 2, x_132); -lean_ctor_set(x_135, 3, x_103); -x_136 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_136, 0, x_135); -lean_ctor_set(x_136, 1, x_1); -lean_ctor_set(x_136, 2, x_2); -x_137 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_137, 0, x_136); -lean_ctor_set(x_137, 1, x_5); -return x_137; +lean_ctor_set(x_135, 1, x_5); +return x_135; } else { -lean_object* x_138; lean_object* x_139; uint8_t x_140; -x_138 = lean_ctor_get(x_100, 2); -lean_inc(x_138); -lean_dec(x_100); -x_139 = lean_ctor_get(x_138, 0); -lean_inc(x_139); -x_140 = lean_nat_dec_le(x_109, x_109); -if (x_140 == 0) +uint8_t x_136; +x_136 = lean_nat_dec_le(x_105, x_105); +if (x_136 == 0) { -lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; -lean_dec(x_109); -lean_dec(x_108); -x_141 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; -if (lean_is_scalar(x_126)) { - x_142 = lean_alloc_ctor(0, 8, 0); +lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; +lean_dec(x_105); +lean_dec(x_104); +x_137 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; +if (lean_is_scalar(x_123)) { + x_138 = lean_alloc_ctor(0, 8, 0); } else { - x_142 = x_126; -} -lean_ctor_set(x_142, 0, x_120); -lean_ctor_set(x_142, 1, x_141); -lean_ctor_set(x_142, 2, x_121); -lean_ctor_set(x_142, 3, x_122); -lean_ctor_set(x_142, 4, x_123); -lean_ctor_set(x_142, 5, x_124); -lean_ctor_set(x_142, 6, x_130); -lean_ctor_set(x_142, 7, x_125); -x_143 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_143, 0, x_142); -lean_ctor_set(x_143, 1, x_138); -lean_ctor_set(x_143, 2, x_139); -lean_ctor_set(x_143, 3, x_103); -x_144 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_144, 0, x_143); -lean_ctor_set(x_144, 1, x_1); -lean_ctor_set(x_144, 2, x_2); -x_145 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_145, 0, x_144); -lean_ctor_set(x_145, 1, x_5); -return x_145; + x_138 = x_123; +} +lean_ctor_set(x_138, 0, x_117); +lean_ctor_set(x_138, 1, x_137); +lean_ctor_set(x_138, 2, x_118); +lean_ctor_set(x_138, 3, x_119); +lean_ctor_set(x_138, 4, x_120); +lean_ctor_set(x_138, 5, x_121); +lean_ctor_set(x_138, 6, x_127); +lean_ctor_set(x_138, 7, x_122); +x_139 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_139, 0, x_138); +lean_ctor_set(x_139, 1, x_128); +lean_ctor_set(x_139, 2, x_129); +lean_ctor_set(x_139, 3, x_130); +x_140 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_140, 0, x_139); +lean_ctor_set(x_140, 1, x_1); +lean_ctor_set(x_140, 2, x_2); +x_141 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_141, 0, x_140); +lean_ctor_set(x_141, 1, x_5); +return x_141; } else { -size_t x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; -x_146 = lean_usize_of_nat(x_109); -lean_dec(x_109); -x_147 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; -x_148 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__5(x_108, x_107, x_146, x_147); -lean_dec(x_108); -if (lean_is_scalar(x_126)) { - x_149 = lean_alloc_ctor(0, 8, 0); +size_t x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; +x_142 = lean_usize_of_nat(x_105); +lean_dec(x_105); +x_143 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; +x_144 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__6(x_104, x_103, x_142, x_143); +lean_dec(x_104); +if (lean_is_scalar(x_123)) { + x_145 = lean_alloc_ctor(0, 8, 0); } else { - x_149 = x_126; -} -lean_ctor_set(x_149, 0, x_120); -lean_ctor_set(x_149, 1, x_148); -lean_ctor_set(x_149, 2, x_121); -lean_ctor_set(x_149, 3, x_122); -lean_ctor_set(x_149, 4, x_123); -lean_ctor_set(x_149, 5, x_124); -lean_ctor_set(x_149, 6, x_130); -lean_ctor_set(x_149, 7, x_125); -x_150 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_150, 0, x_149); -lean_ctor_set(x_150, 1, x_138); -lean_ctor_set(x_150, 2, x_139); -lean_ctor_set(x_150, 3, x_103); -x_151 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_151, 0, x_150); -lean_ctor_set(x_151, 1, x_1); -lean_ctor_set(x_151, 2, x_2); -x_152 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_152, 0, x_151); -lean_ctor_set(x_152, 1, x_5); -return x_152; + x_145 = x_123; +} +lean_ctor_set(x_145, 0, x_117); +lean_ctor_set(x_145, 1, x_144); +lean_ctor_set(x_145, 2, x_118); +lean_ctor_set(x_145, 3, x_119); +lean_ctor_set(x_145, 4, x_120); +lean_ctor_set(x_145, 5, x_121); +lean_ctor_set(x_145, 6, x_127); +lean_ctor_set(x_145, 7, x_122); +x_146 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_146, 0, x_145); +lean_ctor_set(x_146, 1, x_128); +lean_ctor_set(x_146, 2, x_129); +lean_ctor_set(x_146, 3, x_130); +x_147 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_147, 0, x_146); +lean_ctor_set(x_147, 1, x_1); +lean_ctor_set(x_147, 2, x_2); +x_148 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_148, 0, x_147); +lean_ctor_set(x_148, 1, x_5); +return x_148; } } } else { -lean_object* x_153; lean_object* x_154; -lean_dec(x_100); -x_153 = lean_ctor_get(x_101, 0); -lean_inc(x_153); -lean_dec(x_101); -x_154 = lean_ctor_get(x_153, 1); -lean_inc(x_154); -lean_dec(x_153); -x_3 = x_154; -x_4 = x_103; +lean_object* x_149; lean_object* x_150; +lean_dec(x_97); +x_149 = lean_ctor_get(x_98, 0); +lean_inc(x_149); +lean_dec(x_98); +x_150 = lean_ctor_get(x_149, 1); +lean_inc(x_150); +lean_dec(x_149); +x_3 = x_150; +x_4 = x_99; goto _start; } } @@ -2826,7 +2849,19 @@ lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; size_t x_5; lean_object* x_6; +x_4 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__5(x_4, x_5, x_3); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { size_t x_5; size_t x_6; lean_object* x_7; @@ -2834,7 +2869,7 @@ x_5 = lean_unbox_usize(x_2); lean_dec(x_2); x_6 = lean_unbox_usize(x_3); lean_dec(x_3); -x_7 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__5(x_1, x_5, x_6, x_4); +x_7 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__6(x_1, x_5, x_6, x_4); lean_dec(x_1); return x_7; } @@ -3169,7 +3204,28 @@ return x_41; } } } -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_runFrontend___spec__1(lean_object* x_1, size_t x_2, size_t x_3) { +LEAN_EXPORT lean_object* l_Lean_Option_setIfNotSet___at_Lean_Elab_runFrontend___spec__1(lean_object* x_1, lean_object* x_2, uint8_t x_3) { +_start: +{ +lean_object* x_4; uint8_t x_5; +x_4 = lean_ctor_get(x_2, 0); +lean_inc(x_4); +x_5 = l_Lean_KVMap_contains(x_1, x_4); +lean_dec(x_4); +if (x_5 == 0) +{ +lean_object* x_6; +x_6 = l_Lean_Option_set___at_Lean_Elab_Term_withoutMacroStackAtErr___spec__1(x_1, x_2, x_3); +return x_6; +} +else +{ +lean_dec(x_2); +return x_1; +} +} +} +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_runFrontend___spec__2(lean_object* x_1, size_t x_2, size_t x_3) { _start: { uint8_t x_4; @@ -3209,7 +3265,7 @@ return x_13; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_runFrontend___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_Elab_runFrontend___spec__3(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { uint8_t x_5; @@ -3304,7 +3360,7 @@ x_14 = lean_ctor_get(x_2, 0); x_15 = 0; x_16 = lean_usize_of_nat(x_6); lean_dec(x_6); -x_17 = l_Array_anyMUnsafe_any___at_Lean_Elab_runFrontend___spec__1(x_5, x_15, x_16); +x_17 = l_Array_anyMUnsafe_any___at_Lean_Elab_runFrontend___spec__2(x_5, x_15, x_16); lean_dec(x_5); if (x_17 == 0) { @@ -3725,7 +3781,7 @@ x_16 = lean_float_div(x_14, x_15); x_17 = 1; x_18 = l_Lean_Parser_mkInputContext(x_1, x_3, x_17); x_19 = l_Lean_Elab_runFrontend___closed__2; -x_20 = l_Lean_Option_set___at_Lean_Elab_Term_withoutMacroStackAtErr___spec__1(x_2, x_19, x_17); +x_20 = l_Lean_Option_setIfNotSet___at_Lean_Elab_runFrontend___spec__1(x_2, x_19, x_17); x_21 = lean_box_uint32(x_5); lean_inc(x_20); lean_inc(x_4); @@ -3986,7 +4042,7 @@ x_75 = 0; x_76 = lean_usize_of_nat(x_36); lean_dec(x_36); x_77 = l_Lean_Elab_runFrontend___closed__3; -x_78 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_runFrontend___spec__2(x_35, x_75, x_76, x_77); +x_78 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_runFrontend___spec__3(x_35, x_75, x_76, x_77); lean_dec(x_35); x_79 = l_Lean_Server_findModuleRefs(x_56, x_78, x_12, x_12); lean_dec(x_78); @@ -4323,7 +4379,7 @@ x_169 = 0; x_170 = lean_usize_of_nat(x_130); lean_dec(x_130); x_171 = l_Lean_Elab_runFrontend___closed__3; -x_172 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_runFrontend___spec__2(x_129, x_169, x_170, x_171); +x_172 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_runFrontend___spec__3(x_129, x_169, x_170, x_171); lean_dec(x_129); x_173 = l_Lean_Server_findModuleRefs(x_150, x_172, x_12, x_12); lean_dec(x_172); @@ -4424,7 +4480,17 @@ return x_192; } } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_runFrontend___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Option_setIfNotSet___at_Lean_Elab_runFrontend___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_Option_setIfNotSet___at_Lean_Elab_runFrontend___spec__1(x_1, x_2, x_4); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_runFrontend___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { size_t x_4; size_t x_5; uint8_t x_6; lean_object* x_7; @@ -4432,13 +4498,13 @@ x_4 = lean_unbox_usize(x_2); lean_dec(x_2); x_5 = lean_unbox_usize(x_3); lean_dec(x_3); -x_6 = l_Array_anyMUnsafe_any___at_Lean_Elab_runFrontend___spec__1(x_1, x_4, x_5); +x_6 = l_Array_anyMUnsafe_any___at_Lean_Elab_runFrontend___spec__2(x_1, x_4, x_5); lean_dec(x_1); x_7 = lean_box(x_6); return x_7; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_runFrontend___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_Elab_runFrontend___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; @@ -4446,7 +4512,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_runFrontend___spec__2(x_1, x_5, x_6, x_4); +x_7 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_runFrontend___spec__3(x_1, x_5, x_6, x_4); lean_dec(x_1); return x_7; } diff --git a/stage0/stdlib/Lean/Elab/GuardMsgs.c b/stage0/stdlib/Lean/Elab/GuardMsgs.c index 4a536adbfe9d..a7e1274f6b20 100644 --- a/stage0/stdlib/Lean/Elab/GuardMsgs.c +++ b/stage0/stdlib/Lean/Elab/GuardMsgs.c @@ -366,6 +366,7 @@ size_t lean_array_size(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_GuardMsgs_parseGuardMsgsSpec___spec__2___closed__7; static lean_object* l_Lean_Elab_Tactic_GuardMsgs_elabGuardMsgs___lambda__1___closed__4; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_GuardMsgs_parseGuardMsgsSpec___spec__2___closed__4; +lean_object* l_Lean_Elab_pushInfoLeaf___at_Lean_withSetOptionIn___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_io_error_to_string(lean_object*); static lean_object* l_Lean_Diff_diff___at_Lean_Elab_Tactic_GuardMsgs_elabGuardMsgs___spec__3___closed__1; lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); @@ -404,7 +405,6 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_GuardMsg LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_GuardMsgs_MessageOrdering_apply___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_GuardMsgs_guardMsgsCodeAction___rarg___closed__6; static lean_object* l_Lean_PersistentArray_findSomeMAux___at_Lean_Elab_Tactic_GuardMsgs_guardMsgsCodeAction___spec__2___closed__1; -lean_object* l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_expandDeclId___spec__11(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_findSomeMAux___at_Lean_Elab_Tactic_GuardMsgs_guardMsgsCodeAction___spec__2___boxed(lean_object*); static lean_object* l_Lean_Diff_lcs___at_Lean_Elab_Tactic_GuardMsgs_elabGuardMsgs___spec__4___closed__4; LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_Tactic_GuardMsgs_elabGuardMsgs___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -9364,7 +9364,7 @@ lean_ctor_set(x_28, 0, x_102); lean_ctor_set(x_99, 1, x_28); x_103 = lean_alloc_ctor(8, 1, 0); lean_ctor_set(x_103, 0, x_99); -x_104 = l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_expandDeclId___spec__11(x_103, x_4, x_5, x_101); +x_104 = l_Lean_Elab_pushInfoLeaf___at_Lean_withSetOptionIn___spec__3(x_103, x_4, x_5, x_101); lean_dec(x_5); lean_dec(x_4); return x_104; @@ -9385,7 +9385,7 @@ lean_ctor_set(x_108, 0, x_105); lean_ctor_set(x_108, 1, x_28); x_109 = lean_alloc_ctor(8, 1, 0); lean_ctor_set(x_109, 0, x_108); -x_110 = l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_expandDeclId___spec__11(x_109, x_4, x_5, x_106); +x_110 = l_Lean_Elab_pushInfoLeaf___at_Lean_withSetOptionIn___spec__3(x_109, x_4, x_5, x_106); lean_dec(x_5); lean_dec(x_4); return x_110; @@ -9432,7 +9432,7 @@ lean_ctor_set(x_28, 0, x_127); lean_ctor_set(x_124, 1, x_28); x_128 = lean_alloc_ctor(8, 1, 0); lean_ctor_set(x_128, 0, x_124); -x_129 = l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_expandDeclId___spec__11(x_128, x_4, x_5, x_126); +x_129 = l_Lean_Elab_pushInfoLeaf___at_Lean_withSetOptionIn___spec__3(x_128, x_4, x_5, x_126); lean_dec(x_5); lean_dec(x_4); return x_129; @@ -9453,7 +9453,7 @@ lean_ctor_set(x_133, 0, x_130); lean_ctor_set(x_133, 1, x_28); x_134 = lean_alloc_ctor(8, 1, 0); lean_ctor_set(x_134, 0, x_133); -x_135 = l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_expandDeclId___spec__11(x_134, x_4, x_5, x_131); +x_135 = l_Lean_Elab_pushInfoLeaf___at_Lean_withSetOptionIn___spec__3(x_134, x_4, x_5, x_131); lean_dec(x_5); lean_dec(x_4); return x_135; @@ -9526,7 +9526,7 @@ lean_ctor_set(x_157, 0, x_153); lean_ctor_set(x_157, 1, x_28); x_158 = lean_alloc_ctor(8, 1, 0); lean_ctor_set(x_158, 0, x_157); -x_159 = l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_expandDeclId___spec__11(x_158, x_4, x_5, x_154); +x_159 = l_Lean_Elab_pushInfoLeaf___at_Lean_withSetOptionIn___spec__3(x_158, x_4, x_5, x_154); lean_dec(x_5); lean_dec(x_4); return x_159; @@ -9585,7 +9585,7 @@ lean_ctor_set(x_179, 0, x_175); lean_ctor_set(x_179, 1, x_28); x_180 = lean_alloc_ctor(8, 1, 0); lean_ctor_set(x_180, 0, x_179); -x_181 = l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_expandDeclId___spec__11(x_180, x_4, x_5, x_176); +x_181 = l_Lean_Elab_pushInfoLeaf___at_Lean_withSetOptionIn___spec__3(x_180, x_4, x_5, x_176); lean_dec(x_5); lean_dec(x_4); return x_181; @@ -9674,7 +9674,7 @@ lean_ctor_set(x_207, 0, x_203); lean_ctor_set(x_207, 1, x_28); x_208 = lean_alloc_ctor(8, 1, 0); lean_ctor_set(x_208, 0, x_207); -x_209 = l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_expandDeclId___spec__11(x_208, x_4, x_5, x_204); +x_209 = l_Lean_Elab_pushInfoLeaf___at_Lean_withSetOptionIn___spec__3(x_208, x_4, x_5, x_204); lean_dec(x_5); lean_dec(x_4); return x_209; @@ -9738,7 +9738,7 @@ lean_ctor_set(x_230, 0, x_226); lean_ctor_set(x_230, 1, x_28); x_231 = lean_alloc_ctor(8, 1, 0); lean_ctor_set(x_231, 0, x_230); -x_232 = l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_expandDeclId___spec__11(x_231, x_4, x_5, x_227); +x_232 = l_Lean_Elab_pushInfoLeaf___at_Lean_withSetOptionIn___spec__3(x_231, x_4, x_5, x_227); lean_dec(x_5); lean_dec(x_4); return x_232; @@ -9865,7 +9865,7 @@ lean_ctor_set(x_269, 0, x_265); lean_ctor_set(x_269, 1, x_28); x_270 = lean_alloc_ctor(8, 1, 0); lean_ctor_set(x_270, 0, x_269); -x_271 = l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_expandDeclId___spec__11(x_270, x_4, x_5, x_266); +x_271 = l_Lean_Elab_pushInfoLeaf___at_Lean_withSetOptionIn___spec__3(x_270, x_4, x_5, x_266); lean_dec(x_5); lean_dec(x_4); return x_271; @@ -9934,7 +9934,7 @@ lean_ctor_set(x_292, 0, x_288); lean_ctor_set(x_292, 1, x_28); x_293 = lean_alloc_ctor(8, 1, 0); lean_ctor_set(x_293, 0, x_292); -x_294 = l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_expandDeclId___spec__11(x_293, x_4, x_5, x_289); +x_294 = l_Lean_Elab_pushInfoLeaf___at_Lean_withSetOptionIn___spec__3(x_293, x_4, x_5, x_289); lean_dec(x_5); lean_dec(x_4); return x_294; @@ -10347,7 +10347,7 @@ lean_ctor_set(x_413, 0, x_409); lean_ctor_set(x_413, 1, x_28); x_414 = lean_alloc_ctor(8, 1, 0); lean_ctor_set(x_414, 0, x_413); -x_415 = l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_expandDeclId___spec__11(x_414, x_4, x_5, x_410); +x_415 = l_Lean_Elab_pushInfoLeaf___at_Lean_withSetOptionIn___spec__3(x_414, x_4, x_5, x_410); lean_dec(x_5); lean_dec(x_4); return x_415; @@ -10416,7 +10416,7 @@ lean_ctor_set(x_436, 0, x_432); lean_ctor_set(x_436, 1, x_28); x_437 = lean_alloc_ctor(8, 1, 0); lean_ctor_set(x_437, 0, x_436); -x_438 = l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_expandDeclId___spec__11(x_437, x_4, x_5, x_433); +x_438 = l_Lean_Elab_pushInfoLeaf___at_Lean_withSetOptionIn___spec__3(x_437, x_4, x_5, x_433); lean_dec(x_5); lean_dec(x_4); return x_438; @@ -10842,7 +10842,7 @@ lean_ctor_set(x_555, 0, x_550); lean_ctor_set(x_555, 1, x_554); x_556 = lean_alloc_ctor(8, 1, 0); lean_ctor_set(x_556, 0, x_555); -x_557 = l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_expandDeclId___spec__11(x_556, x_4, x_5, x_551); +x_557 = l_Lean_Elab_pushInfoLeaf___at_Lean_withSetOptionIn___spec__3(x_556, x_4, x_5, x_551); lean_dec(x_5); lean_dec(x_4); return x_557; @@ -10912,7 +10912,7 @@ lean_ctor_set(x_579, 0, x_574); lean_ctor_set(x_579, 1, x_578); x_580 = lean_alloc_ctor(8, 1, 0); lean_ctor_set(x_580, 0, x_579); -x_581 = l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_expandDeclId___spec__11(x_580, x_4, x_5, x_575); +x_581 = l_Lean_Elab_pushInfoLeaf___at_Lean_withSetOptionIn___spec__3(x_580, x_4, x_5, x_575); lean_dec(x_5); lean_dec(x_4); return x_581; diff --git a/stage0/stdlib/Lean/Elab/Inductive.c b/stage0/stdlib/Lean/Elab/Inductive.c index 1f22aede29b0..fdc8ebee3762 100644 --- a/stage0/stdlib/Lean/Elab/Inductive.c +++ b/stage0/stdlib/Lean/Elab/Inductive.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Lean.Elab.Inductive -// Imports: Lean.Util.ForEachExprWhere Lean.Util.ReplaceLevel Lean.Util.ReplaceExpr Lean.Util.CollectLevelParams Lean.Meta.Constructions Lean.Meta.CollectFVars Lean.Meta.SizeOf Lean.Meta.Injective Lean.Meta.IndPredBelow Lean.Elab.Command Lean.Elab.ComputedFields Lean.Elab.DefView Lean.Elab.DeclUtil Lean.Elab.Deriving.Basic +// Imports: Lean.Util.ForEachExprWhere Lean.Util.ReplaceLevel Lean.Util.ReplaceExpr Lean.Util.CollectLevelParams Lean.Meta.Constructions Lean.Meta.CollectFVars Lean.Meta.SizeOf Lean.Meta.Injective Lean.Meta.IndPredBelow Lean.Elab.Command Lean.Elab.ComputedFields Lean.Elab.DefView Lean.Elab.DeclUtil Lean.Elab.Deriving.Basic Lean.Elab.DeclarationRange #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -15,25 +15,32 @@ extern "C" { #endif static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams___spec__1___closed__1; static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__1___closed__3; +static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___closed__3; LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses___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_object* l_Lean_Expr_const___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isDomainDefEq___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_string_utf8_extract(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__22___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__1___closed__2; lean_object* l_Lean_Elab_Term_levelMVarToParam(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_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_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__22___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_Command_checkValidCtorModifier___rarg___lambda__3___closed__2; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___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_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__2(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*); +static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__5___boxed(lean_object**); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Command_withScope___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Command_withCtorRef___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam___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_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__3; static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__10; LEAN_EXPORT lean_object* l_Lean_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, 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_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__1; LEAN_EXPORT lean_object* l_Lean_ForEachExprWhere_visit___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__5(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__8; LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUsed___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -41,25 +48,33 @@ lean_object* l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(lean_object static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__3___closed__1; lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Lean_Elab_Command_isMutualInductive(lean_object*); 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_object* lean_mk_empty_array_with_capacity(lean_object*); lean_object* l_Lean_mkAppN(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___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_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabDeclAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instInhabitedElabHeaderResult___closed__3; lean_object* l_Lean_Elab_CommandContextInfo_save___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__10___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__4; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__23; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__18; +static lean_object* l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__2; static lean_object* l_Lean_Elab_Command_checkResultingUniverse___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___at___private_Lean_Elab_Inductive_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_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateParams___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_withSaveInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__4___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_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkFreshLevelMVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___rarg___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__14(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_InductiveView_checkLevelNames___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_mkTypeFor___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_mkSizeOfInstances(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkResultingUniverse(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -68,23 +83,35 @@ static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0_ static lean_object* l_Lean_Elab_Command_instInhabitedCtorView___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___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_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_ElabHeaderResult_checkLevelNames___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*); 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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__6; lean_object* l_Lean_Elab_Command_runTermElabM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_sortDeclLevelParams(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4___closed__2; +LEAN_EXPORT lean_object* l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19(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_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidInductiveModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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_Command_withCtorRef___spec__1___rarg___lambda__2(lean_object*, lean_object*, lean_object*); +extern lean_object* l_Lean_declRangeExt; +static lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Command_isMutualInductive___spec__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkResultUniverse(lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_accLevelAtCtor___closed__7; static lean_object* l_Lean_Elab_Command_shouldInferResultUniverse___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_checkValidCtorModifier___rarg___lambda__3___closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_ElabHeaderResult_checkLevelNames___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__1; static lean_object* l_Lean_Elab_Command_accLevelAtCtor___closed__8; +static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__8___closed__1; static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__1___closed__2; +extern lean_object* l_Lean_maxRecDepthErrorMessage; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__6(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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_InductiveView_checkLevelNames___spec__1___closed__2; +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__5(lean_object*, lean_object*); lean_object* l_Lean_indentD(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_resetMaskAt___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__1___closed__1; @@ -97,48 +124,68 @@ uint8_t l_Lean_Exception_isInterrupt(lean_object*); static lean_object* l_Lean_Elab_Command_checkValidInductiveModifier___rarg___closed__2; lean_object* l_Lean_Elab_Command_getMainModule___rarg(lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_synthesizeSyntheticMVars(uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualInductive___spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_allM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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_Lean_Meta_isExprDefEq(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_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__4(lean_object*, size_t, size_t); +lean_object* l_Lean_FileMap_toPosition(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___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_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___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_Elab_liftMacroM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__10___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_uint64_to_usize(uint64_t); lean_object* l_Lean_Level_addOffsetAux(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1___closed__1; static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_InductiveView_checkLevelNames___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_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___closed__2; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabMutualInductive___spec__14(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_CollectLevelMVars_visitExpr___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_withCtorRef___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_checkValidInductiveModifier___rarg___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe___spec__1(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_Lean_instantiateLevelMVars___at_Lean_Elab_Command_accLevelAtCtor___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_Elab_logException___at_Lean_Elab_Command_elabCommand___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualInductive___spec__4___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__8(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___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* l_Lean_Syntax_getId(lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__4; LEAN_EXPORT lean_object* l_Lean_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___closed__1; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_sort___override(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___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_Command_elabMutualInductive___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__9___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_Lean_MessageData_ofList(lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___closed__2; lean_object* l_Array_toSubarray___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26(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_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__8(lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___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*); static lean_object* l_Lean_Elab_Command_instInhabitedCtorView___closed__3; static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__1___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions(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_inductiveSyntaxToView___spec__24___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_Elab_Command_elabMutualInductive___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__4___closed__2; LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInductive(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_mk_array(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__7(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__6; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__4; uint8_t lean_usize_dec_eq(size_t, size_t); +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__17(lean_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_elabInductiveViewsPostprocessing___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_Command_checkValidInductiveModifier___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls_loop___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__5___closed__2; @@ -147,9 +194,8 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_el lean_object* l_Lean_Syntax_getArgs(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___spec__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_Inductive_0__Lean_Elab_Command_checkLevelNames(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_withCtorRef___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___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_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_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_checkValidCtorModifier___rarg___lambda__1___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__5___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -160,11 +206,13 @@ static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_ 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_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__8; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabMutualInductive(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_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__3___closed__1; lean_object* l_Lean_Expr_bvar___override(lean_object*); lean_object* l_Lean_Elab_Command_elabCommand(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_ForEachExprWhere_initCache; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -179,39 +227,48 @@ LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_In LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4_(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams___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*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_removeUnused___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_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__22___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkResultUniverse___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__2(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___lambda__2___closed__3; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeader___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_fvarId_x21(lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__2; lean_object* l_ReaderT_pure___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__12___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +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_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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_EXPORT lean_object* l_Array_erase___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__3(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___closed__4; static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__3; lean_object* l_Lean_RBNode_insert___at_Lean_NameSet_insert___spec__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___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_Elab_Command_elabClassInductive___closed__3; +lean_object* l_Lean_Syntax_getIdAt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkHeaders(lean_object*, 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_InductiveView_checkLevelNames___spec__1___closed__1; lean_object* l_Lean_Meta_forallTelescopeReducing___at_Lean_Meta_getParamNames___spec__2___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4___closed__5; static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__2; static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__9; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___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_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__2___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams___boxed(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_fixedIndicesToParams___lambda__4___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063_(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__19; +uint8_t l_Lean_Linter_getLinterValue(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___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_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__2(lean_object*, lean_object*, lean_object*, size_t, 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___closed__3; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__5___closed__2; +LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_node5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_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*); @@ -221,35 +278,48 @@ static lean_object* l_Lean_localDeclDependsOnPred___at___private_Lean_Elab_Induc size_t lean_usize_of_nat(lean_object*); lean_object* l_Nat_nextPowerOfTwo_go(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4___closed__6; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__5; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInductives(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_IndPredBelow_mkBelow(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_mkInductiveDecl___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_accLevelAtCtor___closed__10; LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidInductiveModifier(lean_object*); lean_object* l_Lean_stringToMessageData(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__4(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_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__1(lean_object*, lean_object*); +uint8_t l_Lean_MapDeclarationExtension_contains___rarg(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_inductiveSyntaxToView___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*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___closed__3; LEAN_EXPORT uint8_t l_Array_contains___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__6(lean_object*, uint8_t); LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses___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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__5; LEAN_EXPORT lean_object* l_Lean_ForEachExprWhere_visited___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__7(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_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__6; +uint8_t lean_string_dec_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getArity___lambda__1___boxed(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_mkAuxConstructions___closed__7; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___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_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__8___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__7; +static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__2___closed__2; +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabMutualInductive___spec__12___boxed(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_checkResultingUniverses_check___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__3; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInductiveViewsPostprocessing___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_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__2; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___spec__1___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Elab_DeclNameGen_0__Lean_Elab_Command_NameGen_winnowExpr_visit___spec__1(lean_object*, lean_object*); +lean_object* lean_string_utf8_byte_size(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withNewBinderInfos___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___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_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__6___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at___private_Lean_Elab_DeclNameGen_0__Lean_Elab_Command_NameGen_winnowExpr_visit___spec__2(lean_object*); lean_object* l_Lean_CollectLevelParams_main(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__4; +LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11___closed__2; 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_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___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*); @@ -259,46 +329,60 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fi lean_object* l_List_mapTR_loop___at_Lean_mkConstWithLevelParams___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___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_Command_checkValidCtorModifier___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabMutualInductive___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__3___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_hasMVar(lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4___closed__4; +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__10___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_accLevelAtCtor___closed__6; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInductiveViewsPostprocessing___lambda__1(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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectLevelParamsInInductive(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__21; size_t lean_ptr_addr(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Elab_Modifiers_addAttr(lean_object*, lean_object*); lean_object* l_List_appendTR___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__3___boxed(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_inductiveSyntaxToView___closed__5; size_t lean_usize_of_nat(lean_object*); lean_object* l_Lean_throwError___at_Lean_Elab_Term_throwErrorIfErrors___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_Inductive_0__Lean_Elab_Command_eqvFirstTypeResult___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_checkValidCtorModifier___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualInductive___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__7; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__2(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_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___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_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___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_Command_elabInductiveViewsPostprocessing(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_accLevelAtCtor___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_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__6; +static lean_object* l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__5; LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_withLCtx___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___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_Command_shouldInferResultUniverse___closed__2; +static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__3; static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__15; +static lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_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_object*, lean_object*); +static lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__6; +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__21___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_45____closed__3; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__4___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__22; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__4___boxed(lean_object**); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__6; static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4___closed__3; static lean_object* l_Lean_Elab_Command_checkResultingUniverse___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidInductiveModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); 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* lean_replace_expr(lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_ensureNoUnassignedMVars(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -306,18 +390,22 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_ge static lean_object* l_Lean_Elab_Command_accLevelAtCtor___closed__4; uint8_t l_Array_contains___at_Lean_Meta_setMVarUserNamesAt___spec__1(lean_object*, lean_object*); lean_object* lean_st_ref_take(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__25; +static lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__4; +lean_object* l_liftExcept___at_Lean_Elab_liftMacroM___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux(lean_object*, 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_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__20(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_mkInductiveDecl___lambda__4___closed__2; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__4; +lean_object* l_Lean_Elab_expandMacroImpl_x3f(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__6; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; +lean_object* l_Lean_Elab_getDeclarationSelectionRef(lean_object*); uint8_t lean_expr_eqv(lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe___spec__1___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_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*); static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__13; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe___spec__1___closed__2; +lean_object* l_Lean_ResolveName_resolveNamespace(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses___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_Meta_forallBoundedTelescope___at_Lean_Meta_arrowDomainsN___spec__6___rarg(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -329,30 +417,40 @@ static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_ uint64_t lean_uint64_shift_right(uint64_t, uint64_t); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__17; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeader(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__1; lean_object* l_Array_feraseIdx___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_accLevelAtCtor___closed__3; lean_object* l_Lean_SourceInfo_fromRef(lean_object*, uint8_t); +LEAN_EXPORT lean_object* l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___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_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__1___boxed(lean_object*, lean_object*); +uint8_t l_Lean_Elab_Modifiers_isProtected(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_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*); static lean_object* l_Lean_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__2___closed__3; 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*); lean_object* l_Lean_Meta_isType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_MessageData_ofSyntax(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___lambda__1___boxed(lean_object**); +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabMutualInductive___spec__13(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ForEachExprWhere_checked___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_node6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___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*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__2; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__14; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__10(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_nat_div(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__19; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses(lean_object*, 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_elabMutualInductive___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam(lean_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_inductiveSyntaxToView___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_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__5; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___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_Linter_logLintIf___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__25___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_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__5; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___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_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__1___closed__4; @@ -360,6 +458,7 @@ lean_object* l_Lean_registerTraceClass(lean_object*, uint8_t, lean_object*, lean LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_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_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__3; static size_t l_Lean_Elab_Command_instInhabitedElabHeaderResult___closed__4; +lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__13(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUsed___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11___closed__5; static lean_object* l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11___closed__4; @@ -367,14 +466,17 @@ LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__ lean_object* l_Lean_Elab_Command_getRef(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeCompatible___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___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_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___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_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__3; LEAN_EXPORT lean_object* l_Lean_throwError___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*); uint8_t l_Lean_Level_occurs(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instInhabitedCtorView___closed__2; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_InductiveView_checkLevelNames(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkCasesOn(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_fixedIndicesToParams_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*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___closed__2; +static lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2; +lean_object* l_Lean_Elab_toAttributeKind___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg___lambda__1(lean_object*, size_t, 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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); @@ -385,15 +487,19 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_ch 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*); static lean_object* l_Lean_Elab_Command_shouldInferResultUniverse___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go(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*); LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInductiveViews___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofFormat(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27___spec__1___boxed(lean_object*, lean_object*); lean_object* l_Lean_PersistentArray_append___rarg(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__2___closed__1; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInductiveViewsPostprocessing___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_Elab_getBetterRef(lean_object*, lean_object*); uint8_t l_Lean_Expr_isMVar(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_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_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabAttrs___at_Lean_Elab_Command_elabMutualInductive___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls___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_assignLevelMVar___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___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_Command_checkValidInductiveModifier___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); @@ -409,9 +515,13 @@ static lean_object* l_Lean_Elab_Command_instInhabitedElabHeaderResult___closed__ static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___closed__1; lean_object* l_Lean_Expr_forallE___override(lean_object*, lean_object*, lean_object*, uint8_t); lean_object* l_outOfBounds___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInductiveViewsPostprocessing___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_Lean_Elab_Command_liftTermElabM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__10___lambda__3(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_checkUnsafe___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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_List_mapTR_loop___at_Lean_Meta_Match_mkMatcher___spec__6(lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -421,12 +531,12 @@ lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageCo LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_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*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___spec__1(lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkLevelNames___spec__1___closed__1; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__24; +lean_object* l_List_forM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkHeader(lean_object*, lean_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___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_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkIndFVar2Const___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_getOptional_x3f(lean_object*); lean_object* lean_st_mk_ref(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__14; LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___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*); @@ -443,22 +553,26 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fi lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__1___closed__1; LEAN_EXPORT lean_object* l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_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_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__16(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_node3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Elab_applyVisibility___at_Lean_Elab_Term_expandDeclId___spec__5(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_append(lean_object*, lean_object*); static lean_object* l_Lean_Elab_withSaveInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__4___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInductiveViews___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabInductives___spec__1(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__13(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_contains___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__6___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInductiveViews___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView(lean_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_levelMVarToParam_levelMVarToParam_x27(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_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_DerivingClassView_applyHandlers(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__2(lean_object*); +LEAN_EXPORT uint8_t l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__1(lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___rarg___closed__1; extern lean_object* l_Lean_levelZero; LEAN_EXPORT lean_object* l_Lean_Elab_Command_shouldInferResultUniverse(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_checkLevelNames___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__2___boxed(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__4___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___closed__3; @@ -466,7 +580,6 @@ LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__ uint8_t l_Lean_Level_hasMVar(lean_object*); extern lean_object* l_Lean_instInhabitedExpr; LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__7(uint8_t, lean_object*, size_t, size_t); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInductiveViews___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_InfoTree_substitute(lean_object*, lean_object*); lean_object* l_Lean_Meta_mkInjectiveTheorems(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_collectUniverses(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -477,34 +590,47 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_shouldInferRes lean_object* l_Lean_Elab_Command_getCurrMacroScope(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__15(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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__3(uint8_t, uint8_t, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint64_t l_Lean_Expr_hash(lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___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_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__18___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_fixedIndicesToParams___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___closed__4; -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkResultingUniverse___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_lengthTRAux___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_accLevelAtCtor___closed__9; +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__10___lambda__4(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__9(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Syntax_getSepArgs(lean_object*); +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Command_isMutualInductive___spec__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___rarg___lambda__1(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_mkAuxConstructions___spec__1___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__4; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__12; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___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*); uint8_t lean_name_eq(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_withCtorRef(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Command_isMutualInductive___spec__1(lean_object*, size_t, size_t); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_getLevelNames___rarg(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_elabCtors(lean_object*, lean_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_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___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_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabDeclAttrs___at_Lean_Elab_Command_elabMutualInductive___spec__2(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*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___spec__3___boxed(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_applyComputedFields___spec__1___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Term_processDefDeriving___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_shouldInferResultUniverse___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_node2(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__10(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_applyComputedFields___spec__2(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_List_allM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_checkResultingUniverse___closed__3; @@ -515,15 +641,20 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_re static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_45____closed__4; static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___closed__1; static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__5; +static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__2___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getArity(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_updateResultingUniverse___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_Command_withCtorRef___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__5(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_fixedIndicesToParams___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_forallTelescopeCompatibleAux___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_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInductiveViews___lambda__3(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__1; +static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___closed__2; +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__20___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_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_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__17___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_Command_instInhabitedElabHeaderResult___closed__5; LEAN_EXPORT uint8_t l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___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*); @@ -536,31 +667,40 @@ LEAN_EXPORT lean_object* l_Lean_Meta_withNewBinderInfos___at___private_Lean_Elab 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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___lambda__1___closed__2; LEAN_EXPORT lean_object* l_List_foldl___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__3(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_Level_mvarId_x21(lean_object*); static lean_object* l_Lean_Elab_Command_checkValidCtorModifier___rarg___lambda__1___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__1; +static lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__2; LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabMutualInductive___spec__7(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_mk_syntax_ident(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___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_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___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* l_Lean_TSyntax_getDocString(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___closed__1; lean_object* l_Lean_Elab_ComputedFields_setComputedFields(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__11; +lean_object* l_Lean_logAt___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__6; LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___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*); static lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__4___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_withAutoBoundImplicitForbiddenPred___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkLevelNames___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_throwErrorAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__11___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_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__6; +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualInductive___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__8___closed__2; LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__4; 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_object* l_Lean_KVMap_setBool(lean_object*, lean_object*, uint8_t); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInductiveViews___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabClassInductive(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_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_Inductive_0__Lean_Elab_Command_getArrowBinderNames(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instInhabitedInductiveView___closed__1; lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Meta_forallTelescopeCompatibleAux___spec__15___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_mod(size_t, size_t); @@ -568,12 +708,18 @@ static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCto LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___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_withCtorRef___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__3___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___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* l_Lean_addDocString_x27___at_Lean_Elab_Term_expandDeclId___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualInductive___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualInductive___spec__1___lambda__3(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_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__1; lean_object* l_Array_append___rarg(lean_object*, lean_object*); uint8_t l_Lean_Environment_contains(lean_object*, lean_object*); uint8_t l_Lean_Level_geq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__15; +LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__1___boxed(lean_object*); lean_object* l_Lean_MessageData_ofExpr(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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_Lean_Elab_Command_elabInductiveViews___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_PersistentArray_mapM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Option_register___at_Lean_Elab_initFn____x40_Lean_Elab_AutoBound___hyg_6____spec__1(lean_object*, lean_object*, lean_object*, lean_object*); @@ -584,13 +730,15 @@ static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCto LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___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*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses___boxed(lean_object*, lean_object*, 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__3___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_throwError___at_Lean_Meta_mkSimpCongrTheorem___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_withAutoBoundImplicit___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___boxed(lean_object*, lean_object*, lean_object*, lean_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_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___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_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkIndFVar2Const___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_userName(lean_object*); lean_object* l_Array_extract___rarg(lean_object*, lean_object*, lean_object*); @@ -598,11 +746,14 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_instInhabitedCtorView; LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___spec__3(lean_object*, lean_object*, size_t, size_t); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_removeUnused___closed__1; lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withNewBinderInfosImp___rarg(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_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__14(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__6; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkLevelNames___spec__1___closed__2; +static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1; static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__8; +uint8_t l_Lean_Elab_Modifiers_isPrivate(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapMAux___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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_Command_withCtorRef___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___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_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__5; static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -610,11 +761,15 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_co lean_object* l_Lean_Elab_Term_addTermInfo_x27(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__2; LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___spec__1(lean_object*, lean_object*, size_t, size_t); +lean_object* l_Lean_FileMap_leanPosToLspPos(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__14___rarg___closed__1; +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__18(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_Inductive_0__Lean_Elab_Command_checkNumParams___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_Array_erase___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__3___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__4___closed__1; static lean_object* l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__1___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInductiveViews___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_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t l_Lean_Syntax_isToken(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe___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*); @@ -625,26 +780,35 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Induc 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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_addLocalVarInfo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__1___closed__3; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_ElabHeaderResult_checkLevelNames(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*); -static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5; lean_object* l_Lean_mkNoConfusion(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Elab_getOptDerivingClasses(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabInductives___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_Expr_replaceFVars(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__1; lean_object* l_Lean_throwError___rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInductiveViews___lambda__4___boxed__const__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_isMutualInductive___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls_loop(lean_object*); +static lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__2; LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectLevelParamsInInductive___spec__2(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_withCtorRef___rarg___closed__1; extern lean_object* l_Lean_NameSet_empty; +static lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__1; static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__5___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_accLevelAtCtor___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_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___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* l_Lean_Elab_Term_collectUnassignedMVars(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__2(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__8; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753_(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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* l_Lean_Level_getLevelOffset(lean_object*); lean_object* l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabClassInductive___closed__1; uint8_t l_List_beq___at___private_Lean_Declaration_0__Lean_beqConstantVal____x40_Lean_Declaration___hyg_433____spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_45____closed__1; static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1___closed__4; @@ -652,16 +816,23 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fi uint8_t lean_nat_dec_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateParams___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_getResetInfoTrees___at_Lean_Elab_Term_withDeclName___spec__3___rarg(lean_object*, lean_object*); +static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__2___closed__1; +static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_resetMaskAt(lean_object*, lean_object*); lean_object* l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__1___closed__4; lean_object* l_Lean_Meta_getFVarLocalDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInductiveViewsPostprocessing___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___closed__1; LEAN_EXPORT lean_object* l_List_mapM_loop___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_object*); +static lean_object* l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__8___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6(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_withUsed(lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceArrowBinderNames(lean_object*, lean_object*); +lean_object* lean_environment_main_module(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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_Elab_Command_elabInductives___lambda__1(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__1; 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_object* l_Lean_instantiateMVars___at___private_Lean_Meta_Basic_0__Lean_Meta_isClassApp_x3f___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -677,13 +848,15 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Induc LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___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_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_InductiveView_checkLevelNames___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*); lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_withCtorRef___rarg___lambda__1___boxed(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_Lean_throwError___at_Lean_Elab_Command_elabMutualInductive___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___lambda__2(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__16; LEAN_EXPORT lean_object* l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6(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_elabInductiveViews(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*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instInhabitedElabHeaderResult___closed__7; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask(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_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -691,7 +864,8 @@ lean_object* l_Lean_indentExpr(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_BinderInfo_isExplicit(uint8_t); LEAN_EXPORT lean_object* l_List_foldl___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__3___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkLevelNames___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_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__5; +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualInductive___spec__1___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_withCtorRef___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__3___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_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___closed__3; static lean_object* l_Lean_Elab_Command_checkValidCtorModifier___rarg___closed__1; @@ -702,63 +876,83 @@ LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Inductive_0_ lean_object* l_Lean_Syntax_node1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_checkValidCtorModifier___rarg___lambda__2___closed__2; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__3; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___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_Command_accLevel_go(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*); +static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__2___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs(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_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11___closed__1; uint8_t l_Lean_NameSet_contains(lean_object*, lean_object*); +lean_object* l_Lean_Elab_Term_expandDeclId(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__9___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_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__20; static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___spec__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2(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_set(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_accLevelAtCtor___closed__2; LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__1(lean_object*, lean_object*, size_t, size_t); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___closed__2; +LEAN_EXPORT lean_object* l_Lean_Linter_logLintIf___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__25(lean_object*, 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_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__14___rarg___closed__2; LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_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__4(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, 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*, uint8_t, 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_Command_accLevel_go___spec__2___boxed(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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkTypeFor___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_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___closed__3; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams___spec__1___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__10___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); uint64_t lean_uint64_xor(uint64_t, uint64_t); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PersistentHashMap_insert___at_Lean_assignLevelMVar___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__21(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_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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*); +static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidInductiveModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___spec__1___boxed(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_withExplicitToImplicit___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__2; lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_CollectLevelMVars_visitExpr___spec__2(lean_object*); +static lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__2; LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectLevelParamsInInductive___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkIndFVar2Const___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_ResolveName_resolveGlobalName(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_Lean_Elab_Command_withCtorRef___spec__1___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__8(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_getAppFn(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_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___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*); extern lean_object* l_Lean_levelOne; lean_object* l_Array_mkArray1___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__7___boxed__const__1; lean_object* lean_nat_mul(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__1___closed__2; static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___lambda__2___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_eqvFirstTypeResult(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_checkResultingUniverses_check___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabMutualInductive___spec__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Syntax_getRange_x3f(lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg___lambda__4(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkHeaders___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_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27___lambda__1___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__3; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__2___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___boxed(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_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__2___boxed(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_applyComputedFields___spec__3(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_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1(uint8_t, uint8_t, 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*); @@ -766,35 +960,48 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_is LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeCompatible___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___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_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___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_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1___closed__3; +lean_object* l_Lean_Elab_expandOptDeclSig(lean_object*); static lean_object* l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11___closed__3; +extern lean_object* l_Lean_Linter_linter_deprecated; static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__17; lean_object* l_List_foldl___at_Array_appendList___spec__1___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__2___lambda__1(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_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__5; lean_object* l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); lean_object* l_Array_ofSubarray___rarg(lean_object*); uint8_t l_Lean_LocalDecl_binderInfo(lean_object*); LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___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_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls_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*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabMutualInductive___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___closed__4; +extern lean_object* l_Lean_instInhabitedDeclarationRanges; +lean_object* lean_erase_macro_scopes(lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___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_Command_accLevelAtCtor___closed__5; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___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_List_reverse___rarg(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*); lean_object* l_Lean_Elab_Term_withAuxDecl___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__14___rarg(lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__2___closed__2; static lean_object* l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11___closed__6; lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Term_Quotation_getAntiquotationIds___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_accLevel_go___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__22___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_sub(size_t, size_t); lean_object* lean_array_mk(lean_object*); static lean_object* l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__3; +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__12___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_fixedIndicesToParams___lambda__1(lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls_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*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualInductive___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_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___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*); +static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_withNewBinderInfos___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___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_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_ElabHeaderResult_checkLevelNames___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_Elab_Command_checkValidInductiveModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__18; static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; lean_object* l_Lean_Meta_removeUnused(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -802,8 +1009,12 @@ LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_sho lean_object* l_Lean_Level_mkNaryMax(lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4___closed__1; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__13; +LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualInductive___spec__4___lambda__1(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInductiveViewsPostprocessing___lambda__2___boxed__const__1; lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at___private_Lean_Elab_DeclNameGen_0__Lean_Elab_Command_NameGen_winnowExpr_visit___spec__6(lean_object*, lean_object*); lean_object* l_Array_indexOfAux___at___private_Lean_Meta_Constructions_BRecOn_0__Lean_buildBRecOnMinorPremise_go___spec__1(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__3; +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabMutualInductive___spec__7___boxed(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_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__3; @@ -815,13 +1026,16 @@ static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCto LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___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_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__3; 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_checkParamsAndResultType___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_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Level_isMVar(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__24(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_eqvFirstTypeResult___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_45____closed__2; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_elabAttrs___at_Lean_Elab_Command_elabMutualInductive___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); 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_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1(uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -829,8 +1043,11 @@ static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_ lean_object* lean_array_uget(lean_object*, size_t); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___spec__3(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, 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_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__15(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_array_size(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___spec__1(lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabMutualInductive___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__10___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__6___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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_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*); @@ -839,8 +1056,10 @@ static lean_object* l_Lean_Elab_Command_accLevelAtCtor___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeCompatible___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___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_PersistentArray_mapMAux___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeader___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualInductive___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_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_Elab_Command_withCtorRef___rarg___lambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabMutualInductive___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addTrace___at_Lean_Meta_processPostponed_loop___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_accLevelAtCtor___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -851,9 +1070,11 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_ap LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withUsed___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__10; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_bindingBody_x21(lean_object*); +LEAN_EXPORT lean_object* l_Lean_getDocStringText___at_Lean_Elab_Command_elabMutualInductive___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit(lean_object*); LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___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_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__2___rarg___lambda__2(lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*); @@ -861,6 +1082,8 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_el uint8_t l_Lean_Level_isNeverZero(lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__1___boxed(lean_object**); LEAN_EXPORT uint8_t l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__9___lambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___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_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__22___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_getAppArgsAux(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__6; @@ -868,23 +1091,36 @@ LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_ static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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_Command_checkValidCtorModifier___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualInductive___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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__7; +LEAN_EXPORT lean_object* l_Lean_getDocStringText___at_Lean_Elab_Command_elabMutualInductive___spec__11(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabMutualInductive___spec__8(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__10___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_isTracingEnabledFor___at_Lean_Meta_processPostponed_loop___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse(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_withCtorRef___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_getAttributeImpl(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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_Elab_elabAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_contains___at_Lean_Elab_Command_accLevel_go___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUsed___boxed(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__2; static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__5; +static lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Command_instInhabitedInductiveView; lean_object* lean_array_get_size(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___lambda__1(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__5; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__22___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_accLevel_go___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__2(lean_object*, lean_object*, size_t, size_t); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__22___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_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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_Command_accLevelAtCtor___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_Command_instInhabitedElabHeaderResult___closed__6; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__22(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__1; lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -892,10 +1128,15 @@ uint8_t lean_level_eq(lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_shouldInferResultUniverse___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__6; static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__1; +extern lean_object* l_Lean_Elab_unsupportedSyntaxExceptionId; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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*); uint8_t lean_usize_dec_lt(size_t, size_t); +static lean_object* l_Lean_Elab_Command_elabClassInductive___closed__2; static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__12; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateParams(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_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*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Command_accLevel_go___spec__2(lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__5(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*); @@ -913,6 +1154,7 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_shouldInferRes LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isDomainDefEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__9___lambda__1___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__2; +lean_object* l_List_mapTR_loop___at_Lean_compileDecl___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Exception_isRuntime(lean_object*); static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_45____closed__6; @@ -920,6 +1162,9 @@ lean_object* l_Lean_mkConstWithLevelParams___at_Lean_Elab_Term_expandDeclId___sp LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceArrowBinderNames_go___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_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*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__2; +static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ForEachExprWhere_checked___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ForEachExprWhere_visited___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Level_normalize(lean_object*); @@ -927,24 +1172,32 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidInductiveModifier___rarg( uint8_t l_Lean_Expr_isFVar(lean_object*); uint8_t l_Lean_Expr_isForall(lean_object*); LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUsed___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_expandMacros(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_mvarId_x21(lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___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* l_Lean_mkBRecOnOrBInductionOn(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instInhabitedElabHeaderResult___closed__8; LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___lambda__2(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_elabMutualInductive___spec__5(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__1; static lean_object* l_Lean_Elab_Command_checkValidInductiveModifier___rarg___closed__1; +static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__3___closed__1; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); lean_object* l_Lean_MessageData_ofName(lean_object*); +static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__1___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Meta_Constructions_BRecOn_0__Lean_mkBelowOrIBelow(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_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___spec__2(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_expr_instantiate1(lean_object*, lean_object*); lean_object* l___private_Init_Data_Repr_0__Nat_reprFast(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualInductive___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabDeclAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__4; static lean_object* l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__6; static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___lambda__2___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_elabDeclAttrs___at_Lean_Elab_Command_elabMutualInductive___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls___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*); uint8_t l_Lean_Elab_Modifiers_isPartial(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*); @@ -952,6 +1205,7 @@ static lean_object* l_Lean_Elab_Command_shouldInferResultUniverse___closed__1; static lean_object* l_Lean_Elab_Command_checkValidInductiveModifier___rarg___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__2___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_mkRecOn(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__8; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__3(lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -965,6 +1219,7 @@ lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallTelescopeReducingImp lean_object* l_Lean_Expr_collectFVars(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_checkParamsAndResultType(lean_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_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___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_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_removeUnused(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_instInhabitedInductiveType; LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -977,22 +1232,25 @@ static lean_object* l_Lean_Elab_Command_checkValidCtorModifier___rarg___lambda__ LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*); size_t lean_usize_land(size_t, size_t); +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabMutualInductive___spec__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_accLevelAtCtor(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_withSaveInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInductiveViews___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__1; +LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_elabType(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__5___closed__1; static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__4___closed__1; +lean_object* l_ReaderT_pure___at_Lean_Elab_liftMacroM___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__12(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkIndFVar2Const(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkHeader___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_bindTR_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__5(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); 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*); uint8_t l_Array_isEmpty___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabMutualInductive___spec__10(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__4; lean_object* l_Lean_Level_getOffsetAux(lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_withDeclName___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1327,7 +1585,7 @@ x_4 = lean_alloc_closure((void*)(l_Lean_Elab_Command_checkValidInductiveModifier lean_closure_set(x_4, 0, x_3); lean_closure_set(x_4, 1, x_1); lean_closure_set(x_4, 2, x_2); -x_5 = lean_ctor_get_uint8(x_3, sizeof(void*)*2 + 1); +x_5 = lean_ctor_get_uint8(x_3, sizeof(void*)*3 + 1); lean_dec(x_3); if (x_5 == 0) { @@ -1397,7 +1655,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___rarg___lam _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; -x_5 = lean_ctor_get(x_1, 1); +x_5 = lean_ctor_get(x_1, 2); x_6 = lean_array_get_size(x_5); x_7 = lean_unsigned_to_nat(0u); x_8 = lean_nat_dec_eq(x_6, x_7); @@ -1453,7 +1711,7 @@ x_5 = lean_alloc_closure((void*)(l_Lean_Elab_Command_checkValidCtorModifier___ra lean_closure_set(x_5, 0, x_1); lean_closure_set(x_5, 1, x_2); lean_closure_set(x_5, 2, x_3); -x_6 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 3); +x_6 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 3); lean_dec(x_1); if (x_6 == 0) { @@ -1571,7 +1829,7 @@ x_4 = lean_alloc_closure((void*)(l_Lean_Elab_Command_checkValidCtorModifier___ra lean_closure_set(x_4, 0, x_3); lean_closure_set(x_4, 1, x_1); lean_closure_set(x_4, 2, x_2); -x_5 = lean_ctor_get_uint8(x_3, sizeof(void*)*2 + 1); +x_5 = lean_ctor_get_uint8(x_3, sizeof(void*)*3 + 1); lean_dec(x_3); if (x_5 == 0) { @@ -1650,20 +1908,22 @@ return x_2; static lean_object* _init_l_Lean_Elab_Command_instInhabitedCtorView___closed__2() { _start: { -lean_object* x_1; uint8_t x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; +lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; uint8_t x_5; lean_object* x_6; lean_object* x_7; x_1 = lean_box(0); -x_2 = 0; +x_2 = lean_box(0); x_3 = 0; x_4 = 0; -x_5 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; -x_6 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_6, 0, x_1); -lean_ctor_set(x_6, 1, x_5); -lean_ctor_set_uint8(x_6, sizeof(void*)*2, x_2); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 1, x_3); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 2, x_4); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 3, x_3); -return x_6; +x_5 = 0; +x_6 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; +x_7 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_7, 0, x_2); +lean_ctor_set(x_7, 1, x_1); +lean_ctor_set(x_7, 2, x_6); +lean_ctor_set_uint8(x_7, sizeof(void*)*3, x_3); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 1, x_4); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 2, x_5); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 3, x_4); +return x_7; } } static lean_object* _init_l_Lean_Elab_Command_instInhabitedCtorView___closed__3() { @@ -1802,18 +2062,20 @@ return x_2; static lean_object* _init_l_Lean_Elab_Command_instInhabitedElabHeaderResult___closed__8() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Elab_Command_instInhabitedInductiveView___closed__1; -x_2 = l_Lean_Elab_Command_instInhabitedElabHeaderResult___closed__6; -x_3 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; -x_4 = l_Lean_Elab_Command_instInhabitedElabHeaderResult___closed__7; -x_5 = lean_alloc_ctor(0, 5, 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_3); -lean_ctor_set(x_5, 4, x_4); -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 = lean_box(0); +x_2 = l_Lean_Elab_Command_instInhabitedInductiveView___closed__1; +x_3 = l_Lean_Elab_Command_instInhabitedElabHeaderResult___closed__6; +x_4 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; +x_5 = l_Lean_Elab_Command_instInhabitedElabHeaderResult___closed__7; +x_6 = lean_alloc_ctor(0, 6, 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_1); +lean_ctor_set(x_6, 4, x_4); +lean_ctor_set(x_6, 5, x_5); +return x_6; } } static lean_object* _init_l_Lean_Elab_Command_instInhabitedElabHeaderResult() { @@ -1824,1660 +2086,2487 @@ x_1 = l_Lean_Elab_Command_instInhabitedElabHeaderResult___closed__8; return x_1; } } -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___spec__1(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidInductiveModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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: { -uint8_t x_5; -x_5 = lean_usize_dec_eq(x_3, x_4); -if (x_5 == 0) -{ -lean_object* x_6; lean_object* x_7; uint8_t x_8; -x_6 = lean_array_uget(x_2, x_3); -x_7 = lean_ctor_get(x_6, 3); -lean_inc(x_7); -lean_dec(x_6); -x_8 = lean_name_eq(x_7, x_1); -lean_dec(x_7); -if (x_8 == 0) -{ -size_t x_9; size_t x_10; -x_9 = 1; -x_10 = lean_usize_add(x_3, x_9); -x_3 = x_10; -goto _start; -} -else +uint8_t x_10; +x_10 = l_Lean_Elab_Modifiers_isPartial(x_1); +if (x_10 == 0) { -uint8_t x_12; -x_12 = 1; +lean_object* x_11; lean_object* x_12; +lean_dec(x_3); +x_11 = lean_box(0); +x_12 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_11); +lean_ctor_set(x_12, 1, x_9); return x_12; } -} else { -uint8_t x_13; -x_13 = 0; -return x_13; +lean_object* x_13; lean_object* x_14; +x_13 = l_Lean_Elab_Command_checkValidInductiveModifier___rarg___lambda__1___closed__2; +x_14 = l_Lean_throwError___at_Lean_Elab_Term_throwErrorIfErrors___spec__1(x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_14; } } } -LEAN_EXPORT uint8_t l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidInductiveModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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_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_9; +x_9 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 1); +if (x_9 == 0) { -uint8_t x_6; -lean_dec(x_3); -x_6 = 0; -return x_6; +lean_object* x_10; lean_object* x_11; +x_10 = lean_box(0); +x_11 = l_Lean_Elab_Command_checkValidInductiveModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__1(x_1, x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +return x_11; } else { -size_t x_7; size_t x_8; uint8_t x_9; -x_7 = 0; -x_8 = lean_usize_of_nat(x_3); -lean_dec(x_3); -x_9 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___spec__1(x_2, x_1, x_7, x_8); -return x_9; -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ lean_object* x_12; lean_object* x_13; uint8_t x_14; -x_12 = lean_ctor_get(x_7, 1); -x_13 = l_Lean_Meta_getLocalInstances(x_7, x_8, x_9, x_10, x_11); +x_12 = l_Lean_Elab_Command_checkValidInductiveModifier___rarg___closed__2; +x_13 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8); x_14 = !lean_is_exclusive(x_13); if (x_14 == 0) { -lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = lean_ctor_get(x_13, 0); -lean_inc(x_12); -x_16 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_16, 0, x_1); -lean_ctor_set(x_16, 1, x_12); -lean_ctor_set(x_16, 2, x_15); -lean_ctor_set(x_16, 3, x_3); -lean_ctor_set(x_16, 4, x_4); -x_17 = lean_array_push(x_2, x_16); -lean_ctor_set(x_13, 0, x_17); return x_13; } 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_13, 0); -x_19 = lean_ctor_get(x_13, 1); -lean_inc(x_19); -lean_inc(x_18); +lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_15 = lean_ctor_get(x_13, 0); +x_16 = lean_ctor_get(x_13, 1); +lean_inc(x_16); +lean_inc(x_15); lean_dec(x_13); -lean_inc(x_12); -x_20 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_20, 0, x_1); -lean_ctor_set(x_20, 1, x_12); -lean_ctor_set(x_20, 2, x_18); -lean_ctor_set(x_20, 3, x_3); -lean_ctor_set(x_20, 4, x_4); -x_21 = lean_array_push(x_2, x_20); -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_21); -lean_ctor_set(x_22, 1, x_19); -return x_22; -} +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; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__3___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = lean_box(0); -x_2 = lean_array_mk(x_1); -return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -uint8_t x_10; uint8_t x_11; lean_object* x_12; -x_10 = 1; -x_11 = 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_12 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_10, x_11, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_12) == 0) -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_ctor_get(x_12, 1); -lean_inc(x_13); -lean_dec(x_12); -x_14 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__3___closed__1; -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -x_15 = l_Lean_Elab_Term_addAutoBoundImplicits(x_14, x_3, x_4, x_5, x_6, x_7, x_8, x_13); -lean_dec(x_4); -if (lean_obj_tag(x_15) == 0) +uint8_t x_9; lean_object* x_10; +x_9 = 0; +x_10 = l_Lean_Syntax_getRange_x3f(x_1, x_9); +if (lean_obj_tag(x_10) == 0) { -lean_object* x_16; lean_object* x_17; uint8_t x_18; uint8_t x_19; lean_object* 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 = 1; -x_19 = 1; -lean_inc(x_16); -x_20 = l_Lean_Meta_mkForallFVars(x_16, x_1, x_11, x_18, x_19, x_5, x_6, x_7, x_8, x_17); -lean_dec(x_8); -lean_dec(x_7); +lean_object* x_11; lean_object* x_12; lean_dec(x_6); -lean_dec(x_5); -if (lean_obj_tag(x_20) == 0) -{ -uint8_t x_21; -x_21 = !lean_is_exclusive(x_20); -if (x_21 == 0) -{ -lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_22 = lean_ctor_get(x_20, 0); -x_23 = lean_array_get_size(x_16); -lean_dec(x_16); -x_24 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_24, 0, x_22); -lean_ctor_set(x_24, 1, x_23); -lean_ctor_set(x_20, 0, x_24); -return x_20; +x_11 = lean_box(0); +x_12 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_11); +lean_ctor_set(x_12, 1, x_8); +return x_12; } else { -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_20, 0); -x_26 = lean_ctor_get(x_20, 1); -lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_20); -x_27 = lean_array_get_size(x_16); -lean_dec(x_16); -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_29 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_29, 0, x_28); -lean_ctor_set(x_29, 1, x_26); -return x_29; -} -} -else +uint8_t x_13; +x_13 = !lean_is_exclusive(x_10); +if (x_13 == 0) { -uint8_t x_30; +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_14 = lean_ctor_get(x_10, 0); +x_15 = lean_ctor_get(x_6, 1); +lean_inc(x_15); +lean_dec(x_6); +x_16 = lean_ctor_get(x_14, 0); +lean_inc(x_16); +lean_inc(x_15); +x_17 = l_Lean_FileMap_toPosition(x_15, x_16); lean_dec(x_16); -x_30 = !lean_is_exclusive(x_20); -if (x_30 == 0) +x_18 = lean_ctor_get(x_14, 1); +lean_inc(x_18); +lean_dec(x_14); +lean_inc(x_15); +x_19 = l_Lean_FileMap_toPosition(x_15, x_18); +lean_dec(x_18); +lean_inc(x_17); +x_20 = l_Lean_FileMap_leanPosToLspPos(x_15, x_17); +x_21 = !lean_is_exclusive(x_20); +if (x_21 == 0) { +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_22 = lean_ctor_get(x_20, 1); +x_23 = lean_ctor_get(x_20, 0); +lean_dec(x_23); +lean_inc(x_19); +x_24 = l_Lean_FileMap_leanPosToLspPos(x_15, x_19); +lean_dec(x_15); +x_25 = lean_ctor_get(x_24, 1); +lean_inc(x_25); +lean_dec(x_24); +x_26 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_26, 0, x_17); +lean_ctor_set(x_26, 1, x_22); +lean_ctor_set(x_26, 2, x_19); +lean_ctor_set(x_26, 3, x_25); +lean_ctor_set(x_10, 0, x_26); +lean_ctor_set(x_20, 1, x_8); +lean_ctor_set(x_20, 0, x_10); return x_20; } else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_31 = lean_ctor_get(x_20, 0); -x_32 = lean_ctor_get(x_20, 1); -lean_inc(x_32); -lean_inc(x_31); +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_27 = lean_ctor_get(x_20, 1); +lean_inc(x_27); lean_dec(x_20); -x_33 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_33, 0, x_31); -lean_ctor_set(x_33, 1, x_32); -return x_33; -} +lean_inc(x_19); +x_28 = l_Lean_FileMap_leanPosToLspPos(x_15, x_19); +lean_dec(x_15); +x_29 = lean_ctor_get(x_28, 1); +lean_inc(x_29); +lean_dec(x_28); +x_30 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_30, 0, x_17); +lean_ctor_set(x_30, 1, x_27); +lean_ctor_set(x_30, 2, x_19); +lean_ctor_set(x_30, 3, x_29); +lean_ctor_set(x_10, 0, x_30); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_10); +lean_ctor_set(x_31, 1, x_8); +return x_31; } } else { -uint8_t x_34; -lean_dec(x_8); -lean_dec(x_7); +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_32 = lean_ctor_get(x_10, 0); +lean_inc(x_32); +lean_dec(x_10); +x_33 = lean_ctor_get(x_6, 1); +lean_inc(x_33); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_1); -x_34 = !lean_is_exclusive(x_15); -if (x_34 == 0) -{ -return x_15; -} -else -{ -lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_35 = lean_ctor_get(x_15, 0); -x_36 = lean_ctor_get(x_15, 1); +x_34 = lean_ctor_get(x_32, 0); +lean_inc(x_34); +lean_inc(x_33); +x_35 = l_Lean_FileMap_toPosition(x_33, x_34); +lean_dec(x_34); +x_36 = lean_ctor_get(x_32, 1); lean_inc(x_36); +lean_dec(x_32); +lean_inc(x_33); +x_37 = l_Lean_FileMap_toPosition(x_33, x_36); +lean_dec(x_36); lean_inc(x_35); -lean_dec(x_15); -x_37 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -return x_37; -} -} +x_38 = l_Lean_FileMap_leanPosToLspPos(x_33, x_35); +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); } -else -{ -uint8_t x_38; -lean_dec(x_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_38 = !lean_is_exclusive(x_12); -if (x_38 == 0) -{ -return x_12; +lean_inc(x_37); +x_41 = l_Lean_FileMap_leanPosToLspPos(x_33, x_37); +lean_dec(x_33); +x_42 = lean_ctor_get(x_41, 1); +lean_inc(x_42); +lean_dec(x_41); +x_43 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_43, 0, x_35); +lean_ctor_set(x_43, 1, x_39); +lean_ctor_set(x_43, 2, x_37); +lean_ctor_set(x_43, 3, x_42); +x_44 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_44, 0, x_43); +if (lean_is_scalar(x_40)) { + x_45 = lean_alloc_ctor(0, 2, 0); +} else { + x_45 = x_40; } -else -{ -lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_39 = lean_ctor_get(x_12, 0); -x_40 = lean_ctor_get(x_12, 1); -lean_inc(x_40); -lean_inc(x_39); -lean_dec(x_12); -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_ctor_set(x_45, 0, x_44); +lean_ctor_set(x_45, 1, x_8); +return x_45; } } } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__4___closed__1() { +static lean_object* _init_l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("invalid inductive type, resultant type is not a sort", 52, 52); +x_1 = l_Lean_declRangeExt; return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__4___closed__2() { +static lean_object* _init_l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__4___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); +x_1 = l_Lean_Elab_Command_instInhabitedElabHeaderResult___closed__2; +x_2 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_2, 0, x_1); +lean_ctor_set(x_2, 1, x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___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) { +static lean_object* _init_l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__3() { _start: { -lean_object* x_9; -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_2); -lean_inc(x_1); -x_9 = l_Lean_Elab_Term_elabType(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_9) == 0) +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_instInhabitedElabHeaderResult___closed__2; +x_2 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_2, 0, x_1); +lean_ctor_set(x_2, 1, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__4() { +_start: { -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); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_10); -x_12 = l_Lean_Meta_isTypeFormerType(x_10, x_4, x_5, x_6, x_7, x_11); -if (lean_obj_tag(x_12) == 0) +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_instInhabitedElabHeaderResult___closed__2; +x_2 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_2, 0, x_1); +lean_ctor_set(x_2, 1, x_1); +lean_ctor_set(x_2, 2, x_1); +lean_ctor_set(x_2, 3, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__5() { +_start: { -lean_object* x_13; uint8_t x_14; -x_13 = lean_ctor_get(x_12, 0); -lean_inc(x_13); -x_14 = lean_unbox(x_13); -lean_dec(x_13); -if (x_14 == 0) +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__3; +x_2 = l_Lean_Elab_Command_instInhabitedElabHeaderResult___closed__2; +x_3 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__4; +x_4 = lean_alloc_ctor(0, 7, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_2); +lean_ctor_set(x_4, 3, x_2); +lean_ctor_set(x_4, 4, x_2); +lean_ctor_set(x_4, 5, x_3); +lean_ctor_set(x_4, 6, x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: { -lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; -lean_dec(x_10); -x_15 = lean_ctor_get(x_12, 1); -lean_inc(x_15); -lean_dec(x_12); -x_16 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__4___closed__2; -x_17 = l_Lean_throwErrorAt___at___private_Lean_Elab_Binders_0__Lean_Elab_Term_elabBinderViews_loop___spec__1(x_1, x_16, x_2, x_3, x_4, x_5, x_6, x_7, x_15); -lean_dec(x_7); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_18 = !lean_is_exclusive(x_17); -if (x_18 == 0) +lean_object* x_10; uint8_t x_11; +x_10 = lean_st_ref_get(x_8, x_9); +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) { -return x_17; -} -else +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_12 = lean_ctor_get(x_10, 0); +x_13 = lean_ctor_get(x_10, 1); +x_14 = lean_ctor_get(x_12, 0); +lean_inc(x_14); +lean_dec(x_12); +x_15 = l_Lean_instInhabitedDeclarationRanges; +x_16 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__1; +lean_inc(x_1); +x_17 = l_Lean_MapDeclarationExtension_contains___rarg(x_15, x_16, x_14, x_1); +lean_dec(x_14); +if (x_17 == 0) { -lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_19 = lean_ctor_get(x_17, 0); -x_20 = lean_ctor_get(x_17, 1); -lean_inc(x_20); +lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +lean_free_object(x_10); +x_18 = lean_st_ref_take(x_8, x_13); +x_19 = lean_ctor_get(x_18, 0); lean_inc(x_19); -lean_dec(x_17); -x_21 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_21, 0, x_19); -lean_ctor_set(x_21, 1, x_20); -return x_21; -} +x_20 = lean_ctor_get(x_18, 1); +lean_inc(x_20); +lean_dec(x_18); +x_21 = !lean_is_exclusive(x_19); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; +x_22 = lean_ctor_get(x_19, 0); +x_23 = lean_ctor_get(x_19, 4); +lean_dec(x_23); +x_24 = l_Lean_MapDeclarationExtension_insert___rarg(x_16, x_22, x_1, x_2); +x_25 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__2; +lean_ctor_set(x_19, 4, x_25); +lean_ctor_set(x_19, 0, x_24); +x_26 = lean_st_ref_set(x_8, x_19, x_20); +x_27 = lean_ctor_get(x_26, 1); +lean_inc(x_27); +lean_dec(x_26); +x_28 = lean_st_ref_take(x_6, x_27); +x_29 = lean_ctor_get(x_28, 0); +lean_inc(x_29); +x_30 = lean_ctor_get(x_28, 1); +lean_inc(x_30); +lean_dec(x_28); +x_31 = !lean_is_exclusive(x_29); +if (x_31 == 0) +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; +x_32 = lean_ctor_get(x_29, 1); +lean_dec(x_32); +x_33 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__5; +lean_ctor_set(x_29, 1, x_33); +x_34 = lean_st_ref_set(x_6, x_29, x_30); +x_35 = !lean_is_exclusive(x_34); +if (x_35 == 0) +{ +lean_object* x_36; lean_object* x_37; +x_36 = lean_ctor_get(x_34, 0); +lean_dec(x_36); +x_37 = lean_box(0); +lean_ctor_set(x_34, 0, x_37); +return x_34; } else { -lean_object* x_22; lean_object* x_23; lean_object* x_24; -lean_dec(x_1); -x_22 = lean_ctor_get(x_12, 1); -lean_inc(x_22); -lean_dec(x_12); -x_23 = lean_box(0); -x_24 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__3(x_10, x_23, x_2, x_3, x_4, x_5, x_6, x_7, x_22); -return x_24; +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_34, 1); +lean_inc(x_38); +lean_dec(x_34); +x_39 = lean_box(0); +x_40 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_40, 0, x_39); +lean_ctor_set(x_40, 1, x_38); +return x_40; } } else { -uint8_t x_25; -lean_dec(x_10); -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 = !lean_is_exclusive(x_12); -if (x_25 == 0) -{ -return x_12; +lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_41 = lean_ctor_get(x_29, 0); +x_42 = lean_ctor_get(x_29, 2); +x_43 = lean_ctor_get(x_29, 3); +x_44 = lean_ctor_get(x_29, 4); +lean_inc(x_44); +lean_inc(x_43); +lean_inc(x_42); +lean_inc(x_41); +lean_dec(x_29); +x_45 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__5; +x_46 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_46, 0, x_41); +lean_ctor_set(x_46, 1, x_45); +lean_ctor_set(x_46, 2, x_42); +lean_ctor_set(x_46, 3, x_43); +lean_ctor_set(x_46, 4, x_44); +x_47 = lean_st_ref_set(x_6, x_46, x_30); +x_48 = lean_ctor_get(x_47, 1); +lean_inc(x_48); +if (lean_is_exclusive(x_47)) { + lean_ctor_release(x_47, 0); + lean_ctor_release(x_47, 1); + x_49 = x_47; +} else { + lean_dec_ref(x_47); + x_49 = lean_box(0); } -else -{ -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_12, 0); -x_27 = lean_ctor_get(x_12, 1); -lean_inc(x_27); -lean_inc(x_26); -lean_dec(x_12); -x_28 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_28, 0, x_26); -lean_ctor_set(x_28, 1, x_27); -return x_28; +x_50 = lean_box(0); +if (lean_is_scalar(x_49)) { + x_51 = lean_alloc_ctor(0, 2, 0); +} else { + x_51 = x_49; } +lean_ctor_set(x_51, 0, x_50); +lean_ctor_set(x_51, 1, x_48); +return x_51; } } else { -uint8_t x_29; -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_29 = !lean_is_exclusive(x_9); -if (x_29 == 0) -{ -return x_9; +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_52 = lean_ctor_get(x_19, 0); +x_53 = lean_ctor_get(x_19, 1); +x_54 = lean_ctor_get(x_19, 2); +x_55 = lean_ctor_get(x_19, 3); +x_56 = lean_ctor_get(x_19, 5); +x_57 = lean_ctor_get(x_19, 6); +lean_inc(x_57); +lean_inc(x_56); +lean_inc(x_55); +lean_inc(x_54); +lean_inc(x_53); +lean_inc(x_52); +lean_dec(x_19); +x_58 = l_Lean_MapDeclarationExtension_insert___rarg(x_16, x_52, x_1, x_2); +x_59 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__2; +x_60 = lean_alloc_ctor(0, 7, 0); +lean_ctor_set(x_60, 0, x_58); +lean_ctor_set(x_60, 1, x_53); +lean_ctor_set(x_60, 2, x_54); +lean_ctor_set(x_60, 3, x_55); +lean_ctor_set(x_60, 4, x_59); +lean_ctor_set(x_60, 5, x_56); +lean_ctor_set(x_60, 6, x_57); +x_61 = lean_st_ref_set(x_8, x_60, x_20); +x_62 = lean_ctor_get(x_61, 1); +lean_inc(x_62); +lean_dec(x_61); +x_63 = lean_st_ref_take(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); +x_67 = lean_ctor_get(x_64, 2); +lean_inc(x_67); +x_68 = lean_ctor_get(x_64, 3); +lean_inc(x_68); +x_69 = lean_ctor_get(x_64, 4); +lean_inc(x_69); +if (lean_is_exclusive(x_64)) { + lean_ctor_release(x_64, 0); + lean_ctor_release(x_64, 1); + lean_ctor_release(x_64, 2); + lean_ctor_release(x_64, 3); + lean_ctor_release(x_64, 4); + x_70 = x_64; +} else { + lean_dec_ref(x_64); + x_70 = lean_box(0); } -else -{ -lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_30 = lean_ctor_get(x_9, 0); -x_31 = lean_ctor_get(x_9, 1); -lean_inc(x_31); -lean_inc(x_30); -lean_dec(x_9); -x_32 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_32, 0, x_30); -lean_ctor_set(x_32, 1, x_31); -return x_32; +x_71 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__5; +if (lean_is_scalar(x_70)) { + x_72 = lean_alloc_ctor(0, 5, 0); +} else { + x_72 = x_70; } +lean_ctor_set(x_72, 0, x_66); +lean_ctor_set(x_72, 1, x_71); +lean_ctor_set(x_72, 2, x_67); +lean_ctor_set(x_72, 3, x_68); +lean_ctor_set(x_72, 4, x_69); +x_73 = lean_st_ref_set(x_6, x_72, x_65); +x_74 = lean_ctor_get(x_73, 1); +lean_inc(x_74); +if (lean_is_exclusive(x_73)) { + lean_ctor_release(x_73, 0); + lean_ctor_release(x_73, 1); + x_75 = x_73; +} else { + lean_dec_ref(x_73); + x_75 = lean_box(0); } +x_76 = lean_box(0); +if (lean_is_scalar(x_75)) { + x_77 = lean_alloc_ctor(0, 2, 0); +} else { + x_77 = x_75; } +lean_ctor_set(x_77, 0, x_76); +lean_ctor_set(x_77, 1, x_74); +return x_77; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -lean_object* x_13; lean_object* x_14; uint8_t x_15; -x_13 = lean_ctor_get(x_8, 1); -x_14 = l_Lean_Meta_getLocalInstances(x_8, x_9, x_10, x_11, x_12); -x_15 = !lean_is_exclusive(x_14); -if (x_15 == 0) -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_14, 0); -lean_inc(x_13); -x_17 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_17, 0, x_1); -lean_ctor_set(x_17, 1, x_13); -lean_ctor_set(x_17, 2, x_16); -lean_ctor_set(x_17, 3, x_2); -lean_ctor_set(x_17, 4, x_3); -x_18 = lean_array_push(x_4, x_17); -lean_ctor_set(x_14, 0, x_18); -return x_14; } 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_14, 0); -x_20 = lean_ctor_get(x_14, 1); -lean_inc(x_20); -lean_inc(x_19); -lean_dec(x_14); -lean_inc(x_13); -x_21 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_21, 0, x_1); -lean_ctor_set(x_21, 1, x_13); -lean_ctor_set(x_21, 2, x_19); -lean_ctor_set(x_21, 3, x_2); -lean_ctor_set(x_21, 4, x_3); -x_22 = lean_array_push(x_4, x_21); -x_23 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_23, 0, x_22); -lean_ctor_set(x_23, 1, x_20); -return x_23; -} +lean_object* x_78; +lean_dec(x_2); +lean_dec(x_1); +x_78 = lean_box(0); +lean_ctor_set(x_10, 0, x_78); +return x_10; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("header params: ", 15, 15); -return x_1; +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_79 = lean_ctor_get(x_10, 0); +x_80 = lean_ctor_get(x_10, 1); +lean_inc(x_80); +lean_inc(x_79); +lean_dec(x_10); +x_81 = lean_ctor_get(x_79, 0); +lean_inc(x_81); +lean_dec(x_79); +x_82 = l_Lean_instInhabitedDeclarationRanges; +x_83 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__1; +lean_inc(x_1); +x_84 = l_Lean_MapDeclarationExtension_contains___rarg(x_82, x_83, x_81, x_1); +lean_dec(x_81); +if (x_84 == 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; 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; +x_85 = lean_st_ref_take(x_8, x_80); +x_86 = lean_ctor_get(x_85, 0); +lean_inc(x_86); +x_87 = lean_ctor_get(x_85, 1); +lean_inc(x_87); +lean_dec(x_85); +x_88 = lean_ctor_get(x_86, 0); +lean_inc(x_88); +x_89 = lean_ctor_get(x_86, 1); +lean_inc(x_89); +x_90 = lean_ctor_get(x_86, 2); +lean_inc(x_90); +x_91 = lean_ctor_get(x_86, 3); +lean_inc(x_91); +x_92 = lean_ctor_get(x_86, 5); +lean_inc(x_92); +x_93 = lean_ctor_get(x_86, 6); +lean_inc(x_93); +if (lean_is_exclusive(x_86)) { + lean_ctor_release(x_86, 0); + lean_ctor_release(x_86, 1); + lean_ctor_release(x_86, 2); + lean_ctor_release(x_86, 3); + lean_ctor_release(x_86, 4); + lean_ctor_release(x_86, 5); + lean_ctor_release(x_86, 6); + x_94 = x_86; +} else { + lean_dec_ref(x_86); + x_94 = lean_box(0); } +x_95 = l_Lean_MapDeclarationExtension_insert___rarg(x_83, x_88, x_1, x_2); +x_96 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__2; +if (lean_is_scalar(x_94)) { + x_97 = lean_alloc_ctor(0, 7, 0); +} else { + x_97 = x_94; +} +lean_ctor_set(x_97, 0, x_95); +lean_ctor_set(x_97, 1, x_89); +lean_ctor_set(x_97, 2, x_90); +lean_ctor_set(x_97, 3, x_91); +lean_ctor_set(x_97, 4, x_96); +lean_ctor_set(x_97, 5, x_92); +lean_ctor_set(x_97, 6, x_93); +x_98 = lean_st_ref_set(x_8, x_97, x_87); +x_99 = lean_ctor_get(x_98, 1); +lean_inc(x_99); +lean_dec(x_98); +x_100 = lean_st_ref_take(x_6, 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; +} else { + lean_dec_ref(x_101); + x_107 = lean_box(0); } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +x_108 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__5; +if (lean_is_scalar(x_107)) { + x_109 = lean_alloc_ctor(0, 5, 0); +} else { + x_109 = x_107; } +lean_ctor_set(x_109, 0, x_103); +lean_ctor_set(x_109, 1, x_108); +lean_ctor_set(x_109, 2, x_104); +lean_ctor_set(x_109, 3, x_105); +lean_ctor_set(x_109, 4, x_106); +x_110 = lean_st_ref_set(x_6, x_109, x_102); +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_110); + x_112 = lean_box(0); } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked(", type: ", 8, 8); -return x_1; +x_113 = lean_box(0); +if (lean_is_scalar(x_112)) { + x_114 = lean_alloc_ctor(0, 2, 0); +} else { + x_114 = x_112; } +lean_ctor_set(x_114, 0, x_113); +lean_ctor_set(x_114, 1, x_111); +return x_114; } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__4() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__3; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +lean_object* x_115; lean_object* x_116; +lean_dec(x_2); +lean_dec(x_1); +x_115 = lean_box(0); +x_116 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_116, 0, x_115); +lean_ctor_set(x_116, 1, x_80); +return x_116; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_45____closed__3; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; -x_12 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__3; -x_13 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_12, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -x_14 = lean_ctor_get(x_13, 0); -lean_inc(x_14); -x_15 = lean_unbox(x_14); +lean_object* x_11; lean_object* x_12; +lean_inc(x_8); +x_11 = l_Lean_Elab_getDeclarationRange_x3f___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__4(x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +if (lean_obj_tag(x_12) == 0) +{ +uint8_t x_13; +lean_dec(x_8); +lean_dec(x_1); +x_13 = !lean_is_exclusive(x_11); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_11, 0); lean_dec(x_14); -if (x_15 == 0) +x_15 = lean_box(0); +lean_ctor_set(x_11, 0, x_15); +return x_11; +} +else { lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_13, 1); +x_16 = lean_ctor_get(x_11, 1); lean_inc(x_16); -lean_dec(x_13); +lean_dec(x_11); x_17 = lean_box(0); -x_18 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__5(x_1, x_3, x_4, x_2, x_17, x_5, x_6, x_7, x_8, x_9, x_10, x_16); +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set(x_18, 1, x_16); return x_18; } -else -{ -uint8_t x_19; -x_19 = !lean_is_exclusive(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; -x_20 = lean_ctor_get(x_13, 1); -x_21 = lean_ctor_get(x_13, 0); -lean_dec(x_21); -lean_inc(x_3); -x_22 = lean_array_to_list(x_3); -x_23 = lean_box(0); -x_24 = l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(x_22, x_23); -x_25 = l_Lean_MessageData_ofList(x_24); -x_26 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__2; -lean_ctor_set_tag(x_13, 7); -lean_ctor_set(x_13, 1, x_25); -lean_ctor_set(x_13, 0, x_26); -x_27 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__4; -x_28 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_28, 0, x_13); -lean_ctor_set(x_28, 1, x_27); -lean_inc(x_4); -x_29 = l_Lean_MessageData_ofExpr(x_4); -x_30 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_30, 0, x_28); -lean_ctor_set(x_30, 1, x_29); -x_31 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5; -x_32 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_32, 0, x_30); -lean_ctor_set(x_32, 1, x_31); -x_33 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_12, x_32, x_5, x_6, x_7, x_8, x_9, x_10, 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); -x_36 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__5(x_1, x_3, x_4, x_2, x_34, x_5, x_6, x_7, x_8, x_9, x_10, x_35); -lean_dec(x_34); -return x_36; } else { -lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; 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_37 = lean_ctor_get(x_13, 1); -lean_inc(x_37); -lean_dec(x_13); -lean_inc(x_3); -x_38 = lean_array_to_list(x_3); -x_39 = lean_box(0); -x_40 = l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(x_38, x_39); -x_41 = l_Lean_MessageData_ofList(x_40); -x_42 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__2; -x_43 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_43, 0, x_42); -lean_ctor_set(x_43, 1, x_41); -x_44 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__4; -x_45 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_45, 0, x_43); -lean_ctor_set(x_45, 1, x_44); -lean_inc(x_4); -x_46 = l_Lean_MessageData_ofExpr(x_4); -x_47 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_47, 0, x_45); -lean_ctor_set(x_47, 1, x_46); -x_48 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5; -x_49 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_49, 0, x_47); -lean_ctor_set(x_49, 1, x_48); -x_50 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_12, x_49, x_5, x_6, x_7, x_8, x_9, x_10, x_37); -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_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__5(x_1, x_3, x_4, x_2, x_51, x_5, x_6, x_7, x_8, x_9, x_10, x_52); -lean_dec(x_51); -return x_53; -} -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; -x_11 = lean_ctor_get(x_1, 7); -lean_inc(x_11); -if (lean_obj_tag(x_11) == 0) -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; uint8_t x_17; lean_object* x_18; -x_12 = l_Lean_Meta_mkFreshLevelMVar(x_6, x_7, x_8, x_9, x_10); -x_13 = lean_ctor_get(x_12, 0); -lean_inc(x_13); -x_14 = lean_ctor_get(x_12, 1); -lean_inc(x_14); +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_19 = lean_ctor_get(x_11, 1); +lean_inc(x_19); +lean_dec(x_11); +x_20 = lean_ctor_get(x_12, 0); +lean_inc(x_20); lean_dec(x_12); -x_15 = l_Lean_Expr_sort___override(x_13); -x_16 = 1; -x_17 = 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_18 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_16, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_14); -if (lean_obj_tag(x_18) == 0) +x_21 = l_Lean_Elab_getDeclarationRange_x3f___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_19); +x_22 = lean_ctor_get(x_21, 0); +lean_inc(x_22); +if (lean_obj_tag(x_22) == 0) { -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 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__2___boxed), 11, 2); -lean_closure_set(x_20, 0, x_1); -lean_closure_set(x_20, 1, x_2); -x_21 = l_Lean_Elab_Term_addAutoBoundImplicits_x27___rarg(x_3, x_15, x_20, x_4, x_5, x_6, x_7, x_8, x_9, x_19); -return x_21; -} -else +uint8_t x_23; +x_23 = !lean_is_exclusive(x_21); +if (x_23 == 0) { -uint8_t x_22; -lean_dec(x_15); -lean_dec(x_9); +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_21, 1); +x_25 = lean_ctor_get(x_21, 0); +lean_dec(x_25); +lean_inc(x_20); +lean_ctor_set(x_21, 1, x_20); +lean_ctor_set(x_21, 0, x_20); +x_26 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5(x_1, x_21, x_4, x_5, x_6, x_7, x_8, x_9, x_24); lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -x_22 = !lean_is_exclusive(x_18); -if (x_22 == 0) -{ -return x_18; +return x_26; } 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_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_21, 1); +lean_inc(x_27); +lean_dec(x_21); +lean_inc(x_20); +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_20); +lean_ctor_set(x_28, 1, x_20); +x_29 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5(x_1, x_28, x_4, x_5, x_6, x_7, x_8, x_9, x_27); +lean_dec(x_8); +return x_29; } } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_11, 0); -lean_inc(x_26); -lean_dec(x_11); -x_27 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__4), 8, 1); -lean_closure_set(x_27, 0, x_26); -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_28 = l_Lean_Elab_Term_withAutoBoundImplicit___rarg(x_27, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_28) == 0) -{ -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_29 = lean_ctor_get(x_28, 0); -lean_inc(x_29); -x_30 = lean_ctor_get(x_28, 1); -lean_inc(x_30); -lean_dec(x_28); -x_31 = lean_ctor_get(x_29, 0); -lean_inc(x_31); -lean_dec(x_29); -x_32 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___boxed), 11, 2); -lean_closure_set(x_32, 0, x_1); -lean_closure_set(x_32, 1, x_2); -x_33 = l_Lean_Elab_Term_addAutoBoundImplicits_x27___rarg(x_3, x_31, x_32, x_4, x_5, x_6, x_7, x_8, x_9, x_30); -return x_33; -} -else +uint8_t x_30; +x_30 = !lean_is_exclusive(x_21); +if (x_30 == 0) { -uint8_t x_34; -lean_dec(x_9); +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_31 = lean_ctor_get(x_21, 1); +x_32 = lean_ctor_get(x_21, 0); +lean_dec(x_32); +x_33 = lean_ctor_get(x_22, 0); +lean_inc(x_33); +lean_dec(x_22); +lean_ctor_set(x_21, 1, x_33); +lean_ctor_set(x_21, 0, x_20); +x_34 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5(x_1, x_21, x_4, x_5, x_6, x_7, x_8, x_9, x_31); lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -x_34 = !lean_is_exclusive(x_28); -if (x_34 == 0) -{ -return x_28; +return x_34; } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_35 = lean_ctor_get(x_28, 0); -x_36 = lean_ctor_get(x_28, 1); -lean_inc(x_36); +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_35 = lean_ctor_get(x_21, 1); lean_inc(x_35); -lean_dec(x_28); -x_37 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_37, 0, x_35); +lean_dec(x_21); +x_36 = lean_ctor_get(x_22, 0); +lean_inc(x_36); +lean_dec(x_22); +x_37 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_37, 0, x_20); lean_ctor_set(x_37, 1, x_36); -return x_37; +x_38 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5(x_1, x_37, x_4, x_5, x_6, x_7, x_8, x_9, x_35); +lean_dec(x_8); +return x_38; } } } } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___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) { +static lean_object* _init_l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__1() { _start: { -lean_object* x_11; -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -x_11 = l_Lean_Elab_Term_withAutoBoundImplicit___rarg(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_11) == 0) +lean_object* x_1; +x_1 = lean_mk_string_unchecked("null", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2() { +_start: { -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_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 = lean_nat_add(x_2, x_14); -x_16 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux(x_3, x_15, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_13); -return x_16; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } -else +} +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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: { -uint8_t x_17; -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_17 = !lean_is_exclusive(x_11); -if (x_17 == 0) +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_12 = lean_box(0); +lean_inc(x_1); +x_13 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_13, 0, x_1); +lean_ctor_set(x_13, 1, x_12); +x_14 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_14, 0, x_2); +lean_ctor_set(x_14, 1, x_13); +x_15 = lean_array_mk(x_14); +x_16 = lean_box(2); +x_17 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2; +x_18 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_18, 0, x_16); +lean_ctor_set(x_18, 1, x_17); +lean_ctor_set(x_18, 2, x_15); +x_19 = l_Lean_Elab_getDeclarationSelectionRef(x_1); +x_20 = l_Lean_Elab_addDeclarationRangesFromSyntax___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3(x_3, x_18, x_19, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_19); +lean_dec(x_18); +return x_20; +} +} +static lean_object* _init_l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__1() { +_start: { -return x_11; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Parser", 6, 6); +return x_1; } -else +} +static lean_object* _init_l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__2() { +_start: { -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_1; +x_1 = lean_mk_string_unchecked("example", 7, 7); +return x_1; } } +static lean_object* _init_l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; +x_2 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__1; +x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__7; +x_4 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__2; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_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_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; lean_object* x_12; uint8_t x_13; -lean_inc(x_1); -x_11 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__1___boxed), 2, 1); -lean_closure_set(x_11, 0, x_1); -x_12 = lean_array_get_size(x_1); -x_13 = lean_nat_dec_lt(x_2, x_12); -lean_dec(x_12); +lean_inc(x_3); +x_11 = l_Lean_Syntax_getKind(x_3); +x_12 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__3; +x_13 = lean_name_eq(x_11, x_12); +lean_dec(x_11); if (x_13 == 0) { lean_object* x_14; lean_object* x_15; -lean_dec(x_2); -lean_dec(x_1); -x_14 = lean_alloc_closure((void*)(l_ReaderT_pure___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__12___rarg___boxed), 8, 1); -lean_closure_set(x_14, 0, x_3); -x_15 = l_Lean_Elab_Term_withAutoBoundImplicitForbiddenPred___rarg(x_11, x_14, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_14 = lean_box(0); +x_15 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1(x_3, x_2, x_1, x_14, x_4, x_5, x_6, x_7, x_8, x_9, x_10); return x_15; } else { -lean_object* x_16; 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_array_fget(x_1, x_2); -x_17 = lean_ctor_get(x_16, 6); -lean_inc(x_17); -x_18 = l_Lean_Syntax_getArgs(x_17); -lean_dec(x_17); -x_19 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__7___boxed), 10, 2); -lean_closure_set(x_19, 0, x_16); -lean_closure_set(x_19, 1, x_3); -x_20 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabBinders___rarg), 9, 2); -lean_closure_set(x_20, 0, x_18); -lean_closure_set(x_20, 1, x_19); -x_21 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__8___boxed), 10, 3); -lean_closure_set(x_21, 0, x_20); -lean_closure_set(x_21, 1, x_2); -lean_closure_set(x_21, 2, x_1); -x_22 = l_Lean_Elab_Term_withAutoBoundImplicitForbiddenPred___rarg(x_11, x_21, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_22; -} -} -} -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___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; -x_5 = lean_unbox_usize(x_3); +lean_object* x_16; lean_object* x_17; +lean_dec(x_8); 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_Inductive_0__Lean_Elab_Command_elabHeaderAux___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; +x_16 = lean_box(0); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_16); +lean_ctor_set(x_17, 1, x_10); +return x_17; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { +} +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__12(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -uint8_t x_3; lean_object* x_4; -x_3 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__1(x_1, x_2); +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_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_is_exclusive(x_12); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_14 = lean_ctor_get(x_12, 0); +x_15 = lean_ctor_get(x_12, 1); +x_16 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(x_14, x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_15); lean_dec(x_2); -lean_dec(x_1); -x_4 = lean_box(x_3); -return x_4; -} +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_12, 1, x_18); +lean_ctor_set(x_12, 0, x_11); +lean_ctor_set_tag(x_16, 1); +lean_ctor_set(x_16, 0, x_12); +return x_16; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: +else { -lean_object* x_12; -x_12 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -return x_12; +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_12, 1, x_19); +lean_ctor_set(x_12, 0, x_11); +x_21 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_21, 0, x_12); +lean_ctor_set(x_21, 1, x_20); +return x_21; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +else { -lean_object* x_10; -x_10 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_22 = lean_ctor_get(x_12, 0); +x_23 = lean_ctor_get(x_12, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_12); +x_24 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(x_22, x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_23); lean_dec(x_2); -return x_10; +x_25 = lean_ctor_get(x_24, 0); +lean_inc(x_25); +x_26 = lean_ctor_get(x_24, 1); +lean_inc(x_26); +if (lean_is_exclusive(x_24)) { + lean_ctor_release(x_24, 0); + lean_ctor_release(x_24, 1); + x_27 = x_24; +} else { + lean_dec_ref(x_24); + x_27 = lean_box(0); } +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_11); +lean_ctor_set(x_28, 1, x_25); +if (lean_is_scalar(x_27)) { + x_29 = lean_alloc_ctor(1, 2, 0); +} else { + x_29 = x_27; + lean_ctor_set_tag(x_29, 1); } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___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_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_26); +return x_29; +} +} +} +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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) { _start: { -lean_object* x_13; -x_13 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___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); +uint8_t x_10; +x_10 = !lean_is_exclusive(x_7); +if (x_10 == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_7, 5); +x_12 = l_Lean_replaceRef(x_1, x_11); lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); +lean_ctor_set(x_7, 5, x_12); +x_13 = l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__12(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); return x_13; } -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: +else { -lean_object* x_12; -x_12 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); +lean_object* x_14; lean_object* x_15; lean_object* x_16; 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; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_14 = lean_ctor_get(x_7, 0); +x_15 = lean_ctor_get(x_7, 1); +x_16 = lean_ctor_get(x_7, 2); +x_17 = lean_ctor_get(x_7, 3); +x_18 = lean_ctor_get(x_7, 4); +x_19 = lean_ctor_get(x_7, 5); +x_20 = lean_ctor_get(x_7, 6); +x_21 = lean_ctor_get(x_7, 7); +x_22 = lean_ctor_get(x_7, 8); +x_23 = lean_ctor_get(x_7, 9); +x_24 = lean_ctor_get(x_7, 10); +x_25 = lean_ctor_get_uint8(x_7, sizeof(void*)*12); +x_26 = lean_ctor_get(x_7, 11); +x_27 = lean_ctor_get_uint8(x_7, sizeof(void*)*12 + 1); +lean_inc(x_26); +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_inc(x_15); +lean_inc(x_14); lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -return x_12; +x_28 = l_Lean_replaceRef(x_1, x_19); +lean_dec(x_19); +x_29 = lean_alloc_ctor(0, 12, 2); +lean_ctor_set(x_29, 0, x_14); +lean_ctor_set(x_29, 1, x_15); +lean_ctor_set(x_29, 2, x_16); +lean_ctor_set(x_29, 3, x_17); +lean_ctor_set(x_29, 4, x_18); +lean_ctor_set(x_29, 5, x_28); +lean_ctor_set(x_29, 6, x_20); +lean_ctor_set(x_29, 7, x_21); +lean_ctor_set(x_29, 8, x_22); +lean_ctor_set(x_29, 9, x_23); +lean_ctor_set(x_29, 10, x_24); +lean_ctor_set(x_29, 11, x_26); +lean_ctor_set_uint8(x_29, sizeof(void*)*12, x_25); +lean_ctor_set_uint8(x_29, sizeof(void*)*12 + 1, x_27); +x_30 = l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__12(x_2, x_3, x_4, x_5, x_6, x_29, x_8, x_9); +lean_dec(x_29); +return x_30; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +} +static lean_object* _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__1() { _start: { -lean_object* x_11; -x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__7(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_3); -return x_11; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("runtime", 7, 7); +return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___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) { +static lean_object* _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__2() { _start: { -lean_object* x_11; -x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_2); -return x_11; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("maxRecDepth", 11, 11); +return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams___spec__1___closed__1() { +static lean_object* _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("invalid inductive type, number of parameters mismatch in mutually inductive datatypes", 85, 85); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__1; +x_2 = l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__2; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams___spec__1___closed__2() { +static lean_object* _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams___spec__1___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); +x_1 = l_Lean_maxRecDepthErrorMessage; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams___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) { +static lean_object* _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__5() { _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_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; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__4; +x_2 = l_Lean_MessageData_ofFormat(x_1); +return x_2; } -else +} +static lean_object* _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__6() { +_start: { -lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; -lean_dec(x_5); -x_15 = lean_array_uget(x_2, x_4); -x_16 = lean_ctor_get(x_15, 3); -lean_inc(x_16); -x_17 = lean_array_get_size(x_16); -lean_dec(x_16); -x_18 = lean_nat_dec_eq(x_17, x_1); -lean_dec(x_17); -if (x_18 == 0) +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__3; +x_2 = l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__5; +x_3 = lean_alloc_ctor(8, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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) { +_start: { -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_15, 0); -lean_inc(x_19); -lean_dec(x_15); -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); -lean_dec(x_19); -x_21 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams___spec__1___closed__2; -x_22 = l_Lean_throwErrorAt___at_Lean_Elab_Term_Quotation_getAntiquotationIds___spec__1(x_20, x_21, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_20); -x_23 = !lean_is_exclusive(x_22); -if (x_23 == 0) +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__6; +x_10 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_10, 0, x_1); +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_8); +return x_11; +} +} +static lean_object* _init_l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__14___rarg___closed__1() { +_start: { -return x_22; +lean_object* x_1; +x_1 = l_Lean_Elab_unsupportedSyntaxExceptionId; +return x_1; } -else +} +static lean_object* _init_l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__14___rarg___closed__2() { +_start: { -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_22, 0); -x_25 = lean_ctor_get(x_22, 1); -lean_inc(x_25); -lean_inc(x_24); -lean_dec(x_22); -x_26 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_26, 0, x_24); -lean_ctor_set(x_26, 1, x_25); -return x_26; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__14___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_throwUnsupportedSyntax___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__14___rarg(lean_object* x_1) { +_start: { -size_t x_27; size_t x_28; lean_object* x_29; -lean_dec(x_15); -x_27 = 1; -x_28 = lean_usize_add(x_4, x_27); -x_29 = lean_box(0); -x_4 = x_28; -x_5 = x_29; -goto _start; +lean_object* x_2; lean_object* x_3; +x_2 = l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__14___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_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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) { +_start: +{ +lean_object* x_7; +x_7 = lean_alloc_closure((void*)(l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__14___rarg), 1, 0); +return x_7; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams(lean_object* x_1, lean_object* x_2, lean_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_liftMacroM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__10___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_9; lean_object* x_10; uint8_t x_11; size_t x_12; size_t x_13; lean_object* x_14; -x_9 = lean_array_get_size(x_1); -x_10 = lean_unsigned_to_nat(0u); -x_11 = lean_nat_dec_lt(x_10, x_9); -lean_dec(x_9); -x_12 = lean_array_size(x_1); -x_13 = 0; -if (x_11 == 0) +lean_object* x_5; lean_object* x_6; +x_5 = l_Lean_Elab_expandMacroImpl_x3f(x_1, x_2, x_3, x_4); +x_6 = lean_ctor_get(x_5, 0); +lean_inc(x_6); +if (lean_obj_tag(x_6) == 0) { -lean_object* x_28; lean_object* x_29; -x_28 = l_Lean_Elab_Command_instInhabitedElabHeaderResult; -x_29 = l_outOfBounds___rarg(x_28); -x_14 = x_29; -goto block_27; +uint8_t x_7; +x_7 = !lean_is_exclusive(x_5); +if (x_7 == 0) +{ +lean_object* x_8; lean_object* x_9; +x_8 = lean_ctor_get(x_5, 0); +lean_dec(x_8); +x_9 = lean_box(0); +lean_ctor_set(x_5, 0, x_9); +return x_5; } else { -lean_object* x_30; -x_30 = lean_array_fget(x_1, x_10); -x_14 = x_30; -goto block_27; +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_5, 1); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_box(0); +x_12 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_11); +lean_ctor_set(x_12, 1, x_10); +return x_12; } -block_27: +} +else { -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_15 = lean_ctor_get(x_14, 3); +uint8_t x_13; +x_13 = !lean_is_exclusive(x_6); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_6, 0); +x_15 = lean_ctor_get(x_14, 1); lean_inc(x_15); lean_dec(x_14); -x_16 = lean_array_get_size(x_15); -lean_dec(x_15); -x_17 = lean_box(0); -x_18 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams___spec__1(x_16, x_1, x_12, x_13, x_17, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_18) == 0) +if (lean_obj_tag(x_15) == 0) { -uint8_t x_19; -x_19 = !lean_is_exclusive(x_18); -if (x_19 == 0) +lean_object* x_16; uint8_t x_17; +lean_free_object(x_6); +x_16 = lean_ctor_get(x_5, 1); +lean_inc(x_16); +lean_dec(x_5); +x_17 = !lean_is_exclusive(x_15); +if (x_17 == 0) { -lean_object* x_20; -x_20 = lean_ctor_get(x_18, 0); -lean_dec(x_20); -lean_ctor_set(x_18, 0, x_16); +lean_object* x_18; +x_18 = l_liftExcept___at_Lean_Elab_liftMacroM___spec__1(x_15, x_3, x_16); +lean_dec(x_15); return x_18; } else { -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_16); -lean_ctor_set(x_22, 1, x_21); -return x_22; +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 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_20, 0, x_19); +x_21 = l_liftExcept___at_Lean_Elab_liftMacroM___spec__1(x_20, x_3, x_16); +lean_dec(x_20); +return x_21; } } else { -uint8_t x_23; -lean_dec(x_16); -x_23 = !lean_is_exclusive(x_18); +lean_object* x_22; uint8_t x_23; +x_22 = lean_ctor_get(x_5, 1); +lean_inc(x_22); +lean_dec(x_5); +x_23 = !lean_is_exclusive(x_15); if (x_23 == 0) { -return x_18; +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_15, 0); +lean_ctor_set(x_6, 0, x_24); +lean_ctor_set(x_15, 0, x_6); +x_25 = l_liftExcept___at_Lean_Elab_liftMacroM___spec__1(x_15, x_3, x_22); +lean_dec(x_15); +return x_25; } 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; +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_15, 0); +lean_inc(x_26); +lean_dec(x_15); +lean_ctor_set(x_6, 0, x_26); +x_27 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_27, 0, x_6); +x_28 = l_liftExcept___at_Lean_Elab_liftMacroM___spec__1(x_27, x_3, x_22); +lean_dec(x_27); +return x_28; } } } +else +{ +lean_object* x_29; lean_object* x_30; +x_29 = lean_ctor_get(x_6, 0); +lean_inc(x_29); +lean_dec(x_6); +x_30 = lean_ctor_get(x_29, 1); +lean_inc(x_30); +lean_dec(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; +x_31 = lean_ctor_get(x_5, 1); +lean_inc(x_31); +lean_dec(x_5); +x_32 = lean_ctor_get(x_30, 0); +lean_inc(x_32); +if (lean_is_exclusive(x_30)) { + lean_ctor_release(x_30, 0); + x_33 = x_30; +} else { + lean_dec_ref(x_30); + x_33 = lean_box(0); +} +if (lean_is_scalar(x_33)) { + x_34 = lean_alloc_ctor(0, 1, 0); +} else { + x_34 = x_33; } +lean_ctor_set(x_34, 0, x_32); +x_35 = l_liftExcept___at_Lean_Elab_liftMacroM___spec__1(x_34, x_3, x_31); +lean_dec(x_34); +return x_35; } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: +else { -size_t x_13; size_t x_14; lean_object* x_15; -x_13 = lean_unbox_usize(x_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_Elab_Inductive_0__Lean_Elab_Command_checkNumParams___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_11); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_2); -lean_dec(x_1); -return x_15; +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_5, 1); +lean_inc(x_36); +lean_dec(x_5); +x_37 = lean_ctor_get(x_30, 0); +lean_inc(x_37); +if (lean_is_exclusive(x_30)) { + lean_ctor_release(x_30, 0); + x_38 = x_30; +} else { + lean_dec_ref(x_30); + x_38 = lean_box(0); } +x_39 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_39, 0, x_37); +if (lean_is_scalar(x_38)) { + x_40 = lean_alloc_ctor(1, 1, 0); +} else { + x_40 = x_38; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +lean_ctor_set(x_40, 0, x_39); +x_41 = l_liftExcept___at_Lean_Elab_liftMacroM___spec__1(x_40, x_3, x_36); +lean_dec(x_40); +return x_41; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__10___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_9; -x_9 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_7); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -return x_9; +uint8_t x_5; lean_object* x_6; lean_object* x_7; +x_5 = l_Lean_Environment_contains(x_1, x_2); +x_6 = lean_box(x_5); +x_7 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_7, 0, x_6); +lean_ctor_set(x_7, 1, x_4); +return x_7; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe___spec__1___closed__1() { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__10___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_1; -x_1 = lean_mk_string_unchecked("invalid inductive type, cannot mix unsafe and safe declarations in a mutually inductive datatypes", 97, 97); -return x_1; +lean_object* x_7; lean_object* x_8; +x_7 = l_Lean_ResolveName_resolveNamespace(x_1, x_2, x_3, 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_6); +return x_8; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe___spec__1___closed__2() { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__10___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe___spec__1___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +lean_object* x_7; lean_object* x_8; +x_7 = l_Lean_ResolveName_resolveGlobalName(x_1, x_2, x_3, 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_6); +return x_8; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe___spec__1(uint8_t 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_Lean_Elab_liftMacroM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -uint8_t x_13; -x_13 = lean_usize_dec_lt(x_4, x_3); -if (x_13 == 0) -{ -lean_object* x_14; +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; 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_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, 0); +lean_inc(x_12); lean_dec(x_10); -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_26; uint8_t x_27; -lean_dec(x_5); -x_15 = lean_array_uget(x_2, x_4); -x_16 = lean_ctor_get(x_15, 0); +x_13 = lean_ctor_get(x_6, 3); +lean_inc(x_13); +x_14 = lean_ctor_get(x_6, 4); +lean_inc(x_14); +x_15 = lean_ctor_get(x_6, 5); +lean_inc(x_15); +x_16 = lean_ctor_get(x_6, 6); lean_inc(x_16); -lean_dec(x_15); -x_26 = lean_ctor_get(x_16, 2); -lean_inc(x_26); -x_27 = lean_ctor_get_uint8(x_26, sizeof(void*)*2 + 3); -lean_dec(x_26); -if (x_27 == 0) +x_17 = lean_ctor_get(x_6, 7); +lean_inc(x_17); +x_18 = lean_ctor_get(x_6, 10); +lean_inc(x_18); +lean_inc(x_12); +x_19 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__10___lambda__1___boxed), 4, 1); +lean_closure_set(x_19, 0, x_12); +lean_inc(x_16); +x_20 = lean_alloc_closure((void*)(l_ReaderT_pure___at_Lean_Elab_liftMacroM___spec__2___rarg___boxed), 3, 1); +lean_closure_set(x_20, 0, x_16); +lean_inc(x_12); +x_21 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__10___lambda__2___boxed), 4, 1); +lean_closure_set(x_21, 0, x_12); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_12); +x_22 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__10___lambda__3___boxed), 6, 3); +lean_closure_set(x_22, 0, x_12); +lean_closure_set(x_22, 1, x_16); +lean_closure_set(x_22, 2, x_17); +lean_inc(x_12); +x_23 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__10___lambda__4___boxed), 6, 3); +lean_closure_set(x_23, 0, x_12); +lean_closure_set(x_23, 1, x_16); +lean_closure_set(x_23, 2, x_17); +x_24 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_24, 0, x_19); +lean_ctor_set(x_24, 1, x_20); +lean_ctor_set(x_24, 2, x_21); +lean_ctor_set(x_24, 3, x_22); +lean_ctor_set(x_24, 4, x_23); +x_25 = lean_st_ref_get(x_7, x_11); +x_26 = !lean_is_exclusive(x_25); +if (x_26 == 0) { -if (x_1 == 0) +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_27 = lean_ctor_get(x_25, 0); +x_28 = lean_ctor_get(x_25, 1); +x_29 = lean_ctor_get(x_27, 1); +lean_inc(x_29); +lean_dec(x_27); +x_30 = lean_environment_main_module(x_12); +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_18); +lean_ctor_set(x_31, 3, x_13); +lean_ctor_set(x_31, 4, x_14); +lean_ctor_set(x_31, 5, x_15); +x_32 = lean_box(0); +lean_ctor_set(x_25, 1, x_32); +lean_ctor_set(x_25, 0, x_29); +x_33 = lean_apply_2(x_1, x_31, x_25); +if (lean_obj_tag(x_33) == 0) { -size_t x_28; size_t x_29; lean_object* x_30; -lean_dec(x_16); -x_28 = 1; -x_29 = lean_usize_add(x_4, x_28); -x_30 = lean_box(0); -x_4 = x_29; -x_5 = x_30; -goto _start; +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; +x_34 = lean_ctor_get(x_33, 0); +lean_inc(x_34); +x_35 = lean_ctor_get(x_33, 1); +lean_inc(x_35); +lean_dec(x_33); +x_36 = lean_ctor_get(x_35, 0); +lean_inc(x_36); +x_37 = lean_st_ref_take(x_7, x_28); +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_is_exclusive(x_38); +if (x_40 == 0) +{ +lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; +x_41 = lean_ctor_get(x_38, 1); +lean_dec(x_41); +lean_ctor_set(x_38, 1, x_36); +x_42 = lean_st_ref_set(x_7, x_38, x_39); +x_43 = lean_ctor_get(x_42, 1); +lean_inc(x_43); +lean_dec(x_42); +x_44 = lean_ctor_get(x_35, 1); +lean_inc(x_44); +lean_dec(x_35); +x_45 = l_List_reverse___rarg(x_44); +x_46 = l_List_forM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__2(x_45, x_2, x_3, x_4, x_5, x_6, x_7, x_43); +lean_dec(x_6); +lean_dec(x_2); +x_47 = !lean_is_exclusive(x_46); +if (x_47 == 0) +{ +lean_object* x_48; +x_48 = lean_ctor_get(x_46, 0); +lean_dec(x_48); +lean_ctor_set(x_46, 0, x_34); +return x_46; } else { -lean_object* x_32; -x_32 = lean_box(0); -x_17 = x_32; -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 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_50, 0, x_34); +lean_ctor_set(x_50, 1, x_49); +return x_50; } } else { -if (x_1 == 0) -{ -lean_object* x_33; -x_33 = lean_box(0); -x_17 = x_33; -goto block_25; +lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_51 = lean_ctor_get(x_38, 0); +x_52 = lean_ctor_get(x_38, 2); +x_53 = lean_ctor_get(x_38, 3); +x_54 = lean_ctor_get(x_38, 4); +x_55 = lean_ctor_get(x_38, 5); +x_56 = lean_ctor_get(x_38, 6); +lean_inc(x_56); +lean_inc(x_55); +lean_inc(x_54); +lean_inc(x_53); +lean_inc(x_52); +lean_inc(x_51); +lean_dec(x_38); +x_57 = lean_alloc_ctor(0, 7, 0); +lean_ctor_set(x_57, 0, x_51); +lean_ctor_set(x_57, 1, x_36); +lean_ctor_set(x_57, 2, x_52); +lean_ctor_set(x_57, 3, x_53); +lean_ctor_set(x_57, 4, x_54); +lean_ctor_set(x_57, 5, x_55); +lean_ctor_set(x_57, 6, x_56); +x_58 = lean_st_ref_set(x_7, x_57, x_39); +x_59 = lean_ctor_get(x_58, 1); +lean_inc(x_59); +lean_dec(x_58); +x_60 = lean_ctor_get(x_35, 1); +lean_inc(x_60); +lean_dec(x_35); +x_61 = l_List_reverse___rarg(x_60); +x_62 = l_List_forM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__2(x_61, x_2, x_3, x_4, x_5, x_6, x_7, x_59); +lean_dec(x_6); +lean_dec(x_2); +x_63 = lean_ctor_get(x_62, 1); +lean_inc(x_63); +if (lean_is_exclusive(x_62)) { + lean_ctor_release(x_62, 0); + lean_ctor_release(x_62, 1); + x_64 = x_62; +} else { + lean_dec_ref(x_62); + x_64 = lean_box(0); } -else -{ -size_t x_34; size_t x_35; lean_object* x_36; -lean_dec(x_16); -x_34 = 1; -x_35 = lean_usize_add(x_4, x_34); -x_36 = lean_box(0); -x_4 = x_35; -x_5 = x_36; -goto _start; +if (lean_is_scalar(x_64)) { + x_65 = lean_alloc_ctor(0, 2, 0); +} else { + x_65 = x_64; +} +lean_ctor_set(x_65, 0, x_34); +lean_ctor_set(x_65, 1, x_63); +return x_65; } } -block_25: +else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; -lean_dec(x_17); -x_18 = lean_ctor_get(x_16, 0); -lean_inc(x_18); -lean_dec(x_16); -x_19 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe___spec__1___closed__2; -x_20 = l_Lean_throwErrorAt___at_Lean_Elab_Term_Quotation_getAntiquotationIds___spec__1(x_18, x_19, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_18); -x_21 = !lean_is_exclusive(x_20); -if (x_21 == 0) +lean_object* x_66; +x_66 = lean_ctor_get(x_33, 0); +lean_inc(x_66); +lean_dec(x_33); +if (lean_obj_tag(x_66) == 0) { -return x_20; +lean_object* x_67; lean_object* x_68; lean_object* x_69; uint8_t x_70; +x_67 = lean_ctor_get(x_66, 0); +lean_inc(x_67); +x_68 = lean_ctor_get(x_66, 1); +lean_inc(x_68); +lean_dec(x_66); +x_69 = l_Lean_maxRecDepthErrorMessage; +x_70 = lean_string_dec_eq(x_68, x_69); +if (x_70 == 0) +{ +lean_object* x_71; lean_object* x_72; lean_object* x_73; +x_71 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_71, 0, x_68); +x_72 = l_Lean_MessageData_ofFormat(x_71); +x_73 = l_Lean_throwErrorAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__11(x_67, x_72, x_2, x_3, x_4, x_5, x_6, x_7, x_28); +lean_dec(x_67); +return x_73; } else { -lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_22 = lean_ctor_get(x_20, 0); -x_23 = lean_ctor_get(x_20, 1); -lean_inc(x_23); -lean_inc(x_22); -lean_dec(x_20); -x_24 = lean_alloc_ctor(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_74; +lean_dec(x_68); +x_74 = l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13(x_67, x_2, x_3, x_4, x_5, x_6, x_7, x_28); +lean_dec(x_6); +lean_dec(x_2); +return x_74; } } +else +{ +lean_object* x_75; +lean_dec(x_6); +lean_dec(x_2); +x_75 = l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__14___rarg(x_28); +return x_75; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; lean_object* x_10; uint8_t x_11; size_t x_12; size_t x_13; lean_object* x_14; -x_9 = lean_array_get_size(x_1); -x_10 = lean_unsigned_to_nat(0u); -x_11 = lean_nat_dec_lt(x_10, x_9); -lean_dec(x_9); -x_12 = lean_array_size(x_1); -x_13 = 0; -if (x_11 == 0) -{ -lean_object* x_29; lean_object* x_30; -x_29 = l_Lean_Elab_Command_instInhabitedElabHeaderResult; -x_30 = l_outOfBounds___rarg(x_29); -x_14 = x_30; -goto block_28; } else { -lean_object* x_31; -x_31 = lean_array_fget(x_1, x_10); -x_14 = x_31; -goto block_28; +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_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_ctor_get(x_76, 1); +lean_inc(x_78); +lean_dec(x_76); +x_79 = lean_environment_main_module(x_12); +x_80 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_80, 0, x_24); +lean_ctor_set(x_80, 1, x_79); +lean_ctor_set(x_80, 2, x_18); +lean_ctor_set(x_80, 3, x_13); +lean_ctor_set(x_80, 4, x_14); +lean_ctor_set(x_80, 5, x_15); +x_81 = lean_box(0); +x_82 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_82, 0, x_78); +lean_ctor_set(x_82, 1, x_81); +x_83 = lean_apply_2(x_1, x_80, x_82); +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_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; +x_84 = lean_ctor_get(x_83, 0); +lean_inc(x_84); +x_85 = lean_ctor_get(x_83, 1); +lean_inc(x_85); +lean_dec(x_83); +x_86 = lean_ctor_get(x_85, 0); +lean_inc(x_86); +x_87 = lean_st_ref_take(x_7, x_77); +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); +x_90 = lean_ctor_get(x_88, 0); +lean_inc(x_90); +x_91 = lean_ctor_get(x_88, 2); +lean_inc(x_91); +x_92 = lean_ctor_get(x_88, 3); +lean_inc(x_92); +x_93 = lean_ctor_get(x_88, 4); +lean_inc(x_93); +x_94 = lean_ctor_get(x_88, 5); +lean_inc(x_94); +x_95 = lean_ctor_get(x_88, 6); +lean_inc(x_95); +if (lean_is_exclusive(x_88)) { + lean_ctor_release(x_88, 0); + lean_ctor_release(x_88, 1); + lean_ctor_release(x_88, 2); + lean_ctor_release(x_88, 3); + lean_ctor_release(x_88, 4); + lean_ctor_release(x_88, 5); + lean_ctor_release(x_88, 6); + x_96 = x_88; +} else { + lean_dec_ref(x_88); + x_96 = lean_box(0); +} +if (lean_is_scalar(x_96)) { + x_97 = lean_alloc_ctor(0, 7, 0); +} else { + x_97 = x_96; +} +lean_ctor_set(x_97, 0, x_90); +lean_ctor_set(x_97, 1, x_86); +lean_ctor_set(x_97, 2, x_91); +lean_ctor_set(x_97, 3, x_92); +lean_ctor_set(x_97, 4, x_93); +lean_ctor_set(x_97, 5, x_94); +lean_ctor_set(x_97, 6, x_95); +x_98 = lean_st_ref_set(x_7, x_97, x_89); +x_99 = lean_ctor_get(x_98, 1); +lean_inc(x_99); +lean_dec(x_98); +x_100 = lean_ctor_get(x_85, 1); +lean_inc(x_100); +lean_dec(x_85); +x_101 = l_List_reverse___rarg(x_100); +x_102 = l_List_forM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__2(x_101, x_2, x_3, x_4, x_5, x_6, x_7, x_99); +lean_dec(x_6); +lean_dec(x_2); +x_103 = lean_ctor_get(x_102, 1); +lean_inc(x_103); +if (lean_is_exclusive(x_102)) { + lean_ctor_release(x_102, 0); + lean_ctor_release(x_102, 1); + x_104 = x_102; +} else { + lean_dec_ref(x_102); + x_104 = lean_box(0); } -block_28: +if (lean_is_scalar(x_104)) { + x_105 = lean_alloc_ctor(0, 2, 0); +} else { + x_105 = x_104; +} +lean_ctor_set(x_105, 0, x_84); +lean_ctor_set(x_105, 1, x_103); +return x_105; +} +else { -lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; lean_object* x_19; -x_15 = lean_ctor_get(x_14, 0); -lean_inc(x_15); -lean_dec(x_14); -x_16 = lean_ctor_get(x_15, 2); -lean_inc(x_16); -lean_dec(x_15); -x_17 = lean_ctor_get_uint8(x_16, sizeof(void*)*2 + 3); -lean_dec(x_16); -x_18 = lean_box(0); -x_19 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe___spec__1(x_17, x_1, x_12, x_13, x_18, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_19) == 0) +lean_object* x_106; +x_106 = lean_ctor_get(x_83, 0); +lean_inc(x_106); +lean_dec(x_83); +if (lean_obj_tag(x_106) == 0) { -uint8_t x_20; -x_20 = !lean_is_exclusive(x_19); -if (x_20 == 0) +lean_object* x_107; lean_object* x_108; lean_object* x_109; uint8_t x_110; +x_107 = lean_ctor_get(x_106, 0); +lean_inc(x_107); +x_108 = lean_ctor_get(x_106, 1); +lean_inc(x_108); +lean_dec(x_106); +x_109 = l_Lean_maxRecDepthErrorMessage; +x_110 = lean_string_dec_eq(x_108, x_109); +if (x_110 == 0) { -lean_object* x_21; -x_21 = lean_ctor_get(x_19, 0); -lean_dec(x_21); -lean_ctor_set(x_19, 0, x_18); -return x_19; +lean_object* x_111; lean_object* x_112; lean_object* x_113; +x_111 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_111, 0, x_108); +x_112 = l_Lean_MessageData_ofFormat(x_111); +x_113 = l_Lean_throwErrorAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__11(x_107, x_112, x_2, x_3, x_4, x_5, x_6, x_7, x_77); +lean_dec(x_107); +return x_113; } else { -lean_object* x_22; lean_object* x_23; -x_22 = lean_ctor_get(x_19, 1); -lean_inc(x_22); -lean_dec(x_19); -x_23 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_23, 0, x_18); -lean_ctor_set(x_23, 1, x_22); -return x_23; -} +lean_object* x_114; +lean_dec(x_108); +x_114 = l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13(x_107, x_2, x_3, x_4, x_5, x_6, x_7, x_77); +lean_dec(x_6); +lean_dec(x_2); +return x_114; } -else -{ -uint8_t x_24; -x_24 = !lean_is_exclusive(x_19); -if (x_24 == 0) -{ -return x_19; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_19, 0); -x_26 = lean_ctor_get(x_19, 1); -lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_19); -x_27 = lean_alloc_ctor(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_115; +lean_dec(x_6); +lean_dec(x_2); +x_115 = l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__14___rarg(x_77); +return x_115; } } } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe___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_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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) { _start: { -uint8_t x_13; size_t x_14; size_t x_15; lean_object* x_16; -x_13 = lean_unbox(x_1); -lean_dec(x_1); -x_14 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_15 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_16 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe___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_11); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); +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_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_is_exclusive(x_12); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_14 = lean_ctor_get(x_12, 0); +x_15 = lean_ctor_get(x_12, 1); +x_16 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(x_14, x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_15); lean_dec(x_2); +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_12, 1, x_18); +lean_ctor_set(x_12, 0, x_11); +lean_ctor_set_tag(x_16, 1); +lean_ctor_set(x_16, 0, x_12); 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_12, 1, x_19); +lean_ctor_set(x_12, 0, x_11); +x_21 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_21, 0, x_12); +lean_ctor_set(x_21, 1, x_20); +return x_21; +} } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +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; +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 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(x_22, x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_23); +lean_dec(x_2); +x_25 = lean_ctor_get(x_24, 0); +lean_inc(x_25); +x_26 = lean_ctor_get(x_24, 1); +lean_inc(x_26); +if (lean_is_exclusive(x_24)) { + lean_ctor_release(x_24, 0); + lean_ctor_release(x_24, 1); + x_27 = x_24; +} else { + lean_dec_ref(x_24); + x_27 = lean_box(0); +} +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_11); +lean_ctor_set(x_28, 1, x_25); +if (lean_is_scalar(x_27)) { + x_29 = lean_alloc_ctor(1, 2, 0); +} else { + x_29 = x_27; + lean_ctor_set_tag(x_29, 1); +} +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_26); +return x_29; +} +} +} +static lean_object* _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__1___closed__1() { _start: { -lean_object* x_9; -x_9 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_7); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -return x_9; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Term", 4, 4); +return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkLevelNames___spec__1___closed__1() { +static lean_object* _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__1___closed__2() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("invalid inductive type, universe parameters mismatch in mutually inductive datatypes", 84, 84); +x_1 = lean_mk_string_unchecked("byTactic", 8, 8); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkLevelNames___spec__1___closed__2() { +static lean_object* _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__1___closed__3() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkLevelNames___spec__1___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; +x_2 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__1; +x_3 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__1___closed__1; +x_4 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__1___closed__2; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkLevelNames___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) { +LEAN_EXPORT uint8_t l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__1(lean_object* x_1) { _start: { -uint8_t x_13; -x_13 = lean_usize_dec_lt(x_4, x_3); -if (x_13 == 0) +lean_object* x_2; uint8_t x_3; +x_2 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__1___closed__3; +x_3 = lean_name_eq(x_1, x_2); +if (x_3 == 0) { -lean_object* x_14; -lean_dec(x_10); -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; +uint8_t x_4; +x_4 = 1; +return x_4; } else { -lean_object* x_15; lean_object* x_16; uint8_t x_17; -lean_dec(x_5); -x_15 = lean_array_uget(x_2, x_4); -x_16 = lean_ctor_get(x_15, 5); -lean_inc(x_16); -x_17 = l_List_beq___at___private_Lean_Declaration_0__Lean_beqConstantVal____x40_Lean_Declaration___hyg_433____spec__1(x_16, x_1); -lean_dec(x_16); -if (x_17 == 0) -{ -lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; -x_18 = lean_ctor_get(x_15, 0); -lean_inc(x_18); -lean_dec(x_15); -x_19 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkLevelNames___spec__1___closed__2; -x_20 = l_Lean_throwErrorAt___at_Lean_Elab_Term_Quotation_getAntiquotationIds___spec__1(x_18, x_19, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_18); -x_21 = !lean_is_exclusive(x_20); -if (x_21 == 0) +uint8_t x_5; +x_5 = 0; +return x_5; +} +} +} +static lean_object* _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__2___closed__1() { +_start: { -return x_20; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("unknown attribute [", 19, 19); +return x_1; } -else +} +static lean_object* _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__2___closed__2() { +_start: { -lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_22 = lean_ctor_get(x_20, 0); -x_23 = lean_ctor_get(x_20, 1); -lean_inc(x_23); -lean_inc(x_22); -lean_dec(x_20); -x_24 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_24, 0, x_22); -lean_ctor_set(x_24, 1, x_23); -return x_24; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__2___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -else +static lean_object* _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__2___closed__3() { +_start: { -size_t x_25; size_t x_26; lean_object* x_27; -lean_dec(x_15); -x_25 = 1; -x_26 = lean_usize_add(x_4, x_25); -x_27 = lean_box(0); -x_4 = x_26; -x_5 = x_27; -goto _start; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("]", 1, 1); +return x_1; } } +static lean_object* _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__2___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__2___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkLevelNames(lean_object* x_1, lean_object* x_2, lean_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_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___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, lean_object* x_10) { _start: { -lean_object* x_9; lean_object* x_10; uint8_t x_11; -x_9 = lean_array_get_size(x_1); -x_10 = lean_unsigned_to_nat(1u); -x_11 = lean_nat_dec_lt(x_10, x_9); -if (x_11 == 0) +lean_object* x_11; uint8_t x_12; +x_11 = lean_st_ref_get(x_9, x_10); +x_12 = !lean_is_exclusive(x_11); +if (x_12 == 0) { -lean_object* x_12; lean_object* x_13; -lean_dec(x_9); -lean_dec(x_6); +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_13 = lean_ctor_get(x_11, 0); +x_14 = lean_ctor_get(x_11, 1); +x_15 = lean_ctor_get(x_13, 0); +lean_inc(x_15); +lean_dec(x_13); +lean_inc(x_3); +x_16 = l_Lean_getAttributeImpl(x_15, x_3); +lean_dec(x_15); +if (lean_obj_tag(x_16) == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +lean_dec(x_16); +lean_free_object(x_11); lean_dec(x_2); -x_12 = lean_box(0); -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_12); -lean_ctor_set(x_13, 1, x_8); -return x_13; +x_17 = l_Lean_MessageData_ofName(x_3); +x_18 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__2___closed__2; +x_19 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set(x_19, 1, x_17); +x_20 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__2___closed__4; +x_21 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_21, 0, x_19); +lean_ctor_set(x_21, 1, x_20); +x_22 = l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__15(x_21, x_4, x_5, x_6, x_7, x_8, x_9, x_14); +return x_22; } else { -lean_object* x_14; uint8_t x_15; size_t x_16; size_t x_17; lean_object* x_18; -x_14 = lean_unsigned_to_nat(0u); -x_15 = lean_nat_dec_lt(x_14, x_9); -lean_dec(x_9); -x_16 = lean_array_size(x_1); -x_17 = 0; -if (x_15 == 0) +lean_object* x_23; +lean_dec(x_16); +lean_dec(x_4); +x_23 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_23, 0, x_3); +lean_ctor_set(x_23, 1, x_2); +lean_ctor_set_uint8(x_23, sizeof(void*)*2, x_1); +lean_ctor_set(x_11, 0, x_23); +return x_11; +} +} +else { -lean_object* x_31; lean_object* x_32; -x_31 = l_Lean_Elab_Command_instInhabitedInductiveView; -x_32 = l_outOfBounds___rarg(x_31); -x_18 = x_32; -goto block_30; +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_24 = lean_ctor_get(x_11, 0); +x_25 = lean_ctor_get(x_11, 1); +lean_inc(x_25); +lean_inc(x_24); +lean_dec(x_11); +x_26 = lean_ctor_get(x_24, 0); +lean_inc(x_26); +lean_dec(x_24); +lean_inc(x_3); +x_27 = l_Lean_getAttributeImpl(x_26, x_3); +lean_dec(x_26); +if (lean_obj_tag(x_27) == 0) +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +lean_dec(x_27); +lean_dec(x_2); +x_28 = l_Lean_MessageData_ofName(x_3); +x_29 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__2___closed__2; +x_30 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_30, 0, x_29); +lean_ctor_set(x_30, 1, x_28); +x_31 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__2___closed__4; +x_32 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_31); +x_33 = l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__15(x_32, x_4, x_5, x_6, x_7, x_8, x_9, x_25); +return x_33; } else { -lean_object* x_33; -x_33 = lean_array_fget(x_1, x_14); -x_18 = x_33; -goto block_30; +lean_object* x_34; lean_object* x_35; +lean_dec(x_27); +lean_dec(x_4); +x_34 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_34, 0, x_3); +lean_ctor_set(x_34, 1, x_2); +lean_ctor_set_uint8(x_34, sizeof(void*)*2, x_1); +x_35 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_35, 0, x_34); +lean_ctor_set(x_35, 1, x_25); +return x_35; } -block_30: +} +} +} +static lean_object* _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__1() { +_start: { -lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_19 = lean_ctor_get(x_18, 5); -lean_inc(x_19); -lean_dec(x_18); -x_20 = lean_box(0); -x_21 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkLevelNames___spec__1(x_19, x_1, x_16, x_17, x_20, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__1___boxed), 1, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Attr", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("simple", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___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_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; +x_2 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__1; +x_3 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__2; +x_4 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__3; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("unknown attribute", 17, 17); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__5; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_9 = lean_unsigned_to_nat(0u); +x_10 = l_Lean_Syntax_getArg(x_1, x_9); +x_11 = lean_alloc_closure((void*)(l_Lean_Elab_toAttributeKind___boxed), 3, 1); +lean_closure_set(x_11, 0, x_10); +lean_inc(x_6); +lean_inc(x_2); +x_12 = l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__10(x_11, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +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; +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_unsigned_to_nat(1u); +x_16 = l_Lean_Syntax_getArg(x_1, x_15); +x_17 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__1; +x_18 = lean_alloc_closure((void*)(l_Lean_expandMacros), 4, 2); +lean_closure_set(x_18, 0, x_16); +lean_closure_set(x_18, 1, x_17); +lean_inc(x_6); +lean_inc(x_2); +x_19 = l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__9(x_18, x_2, x_3, x_4, x_5, x_6, x_7, x_14); +if (lean_obj_tag(x_19) == 0) +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_19, 1); +lean_inc(x_21); lean_dec(x_19); -if (lean_obj_tag(x_21) == 0) +lean_inc(x_20); +x_22 = l_Lean_Syntax_getKind(x_20); +x_23 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__4; +x_24 = lean_name_eq(x_22, x_23); +if (x_24 == 0) { -uint8_t x_22; -x_22 = !lean_is_exclusive(x_21); -if (x_22 == 0) +if (lean_obj_tag(x_22) == 1) { -lean_object* x_23; -x_23 = lean_ctor_get(x_21, 0); -lean_dec(x_23); -lean_ctor_set(x_21, 0, x_20); -return x_21; +lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; lean_object* x_29; +x_25 = lean_ctor_get(x_22, 1); +lean_inc(x_25); +lean_dec(x_22); +x_26 = lean_box(0); +x_27 = l_Lean_Name_str___override(x_26, x_25); +x_28 = lean_unbox(x_13); +lean_dec(x_13); +x_29 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__2(x_28, x_20, x_27, x_2, x_3, x_4, x_5, x_6, x_7, x_21); +lean_dec(x_6); +return x_29; } else { -lean_object* x_24; lean_object* x_25; -x_24 = lean_ctor_get(x_21, 1); -lean_inc(x_24); -lean_dec(x_21); -x_25 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_25, 0, x_20); -lean_ctor_set(x_25, 1, x_24); -return x_25; +lean_object* x_30; lean_object* x_31; uint8_t x_32; +lean_dec(x_22); +lean_dec(x_13); +x_30 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__6; +x_31 = l_Lean_throwErrorAt___at_Lean_Elab_Term_processDefDeriving___spec__2(x_20, x_30, x_2, x_3, x_4, x_5, x_6, x_7, x_21); +lean_dec(x_20); +x_32 = !lean_is_exclusive(x_31); +if (x_32 == 0) +{ +return x_31; +} +else +{ +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_31, 0); +x_34 = lean_ctor_get(x_31, 1); +lean_inc(x_34); +lean_inc(x_33); +lean_dec(x_31); +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +return x_35; +} } } else { -uint8_t x_26; -x_26 = !lean_is_exclusive(x_21); -if (x_26 == 0) +lean_object* x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; lean_object* x_40; +lean_dec(x_22); +x_36 = l_Lean_Syntax_getArg(x_20, x_9); +x_37 = l_Lean_Syntax_getId(x_36); +lean_dec(x_36); +x_38 = lean_erase_macro_scopes(x_37); +x_39 = lean_unbox(x_13); +lean_dec(x_13); +x_40 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__2(x_39, x_20, x_38, x_2, x_3, x_4, x_5, x_6, x_7, x_21); +lean_dec(x_6); +return x_40; +} +} +else { -return x_21; +uint8_t x_41; +lean_dec(x_13); +lean_dec(x_6); +lean_dec(x_2); +x_41 = !lean_is_exclusive(x_19); +if (x_41 == 0) +{ +return x_19; } else { -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_21, 0); -x_28 = lean_ctor_get(x_21, 1); -lean_inc(x_28); -lean_inc(x_27); -lean_dec(x_21); -x_29 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_29, 0, x_27); -lean_ctor_set(x_29, 1, x_28); -return x_29; +lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_42 = lean_ctor_get(x_19, 0); +x_43 = lean_ctor_get(x_19, 1); +lean_inc(x_43); +lean_inc(x_42); +lean_dec(x_19); +x_44 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_44, 0, x_42); +lean_ctor_set(x_44, 1, x_43); +return x_44; } } } +else +{ +uint8_t x_45; +lean_dec(x_6); +lean_dec(x_2); +x_45 = !lean_is_exclusive(x_12); +if (x_45 == 0) +{ +return x_12; +} +else +{ +lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_46 = lean_ctor_get(x_12, 0); +x_47 = lean_ctor_get(x_12, 1); +lean_inc(x_47); +lean_inc(x_46); +lean_dec(x_12); +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_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkLevelNames___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_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _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); +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_9); +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; lean_object* x_27; uint8_t x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +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 = lean_ctor_get_uint8(x_9, sizeof(void*)*12); +x_27 = lean_ctor_get(x_9, 11); +lean_inc(x_27); +x_28 = lean_ctor_get_uint8(x_9, sizeof(void*)*12 + 1); +x_29 = l_Lean_replaceRef(x_14, x_20); +lean_dec(x_20); +x_30 = lean_alloc_ctor(0, 12, 2); +lean_ctor_set(x_30, 0, x_15); +lean_ctor_set(x_30, 1, x_16); +lean_ctor_set(x_30, 2, x_17); +lean_ctor_set(x_30, 3, x_18); +lean_ctor_set(x_30, 4, x_19); +lean_ctor_set(x_30, 5, x_29); +lean_ctor_set(x_30, 6, x_21); +lean_ctor_set(x_30, 7, x_22); +lean_ctor_set(x_30, 8, x_23); +lean_ctor_set(x_30, 9, x_24); +lean_ctor_set(x_30, 10, x_25); +lean_ctor_set(x_30, 11, x_27); +lean_ctor_set_uint8(x_30, sizeof(void*)*12, x_26); +lean_ctor_set_uint8(x_30, sizeof(void*)*12 + 1, x_28); +lean_inc(x_5); +x_31 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9(x_14, x_5, x_6, x_7, x_8, x_30, x_10, x_11); +lean_dec(x_14); +if (lean_obj_tag(x_31) == 0) +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; size_t x_35; size_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_array_push(x_4, x_32); +x_35 = 1; +x_36 = lean_usize_add(x_3, x_35); +x_3 = x_36; +x_4 = x_34; +x_11 = x_33; +goto _start; +} +else +{ +uint8_t x_38; +x_38 = !lean_is_exclusive(x_31); +if (x_38 == 0) +{ +lean_object* x_39; lean_object* x_40; uint8_t x_41; +x_39 = lean_ctor_get(x_31, 0); +x_40 = lean_ctor_get(x_31, 1); +x_41 = l_Lean_Exception_isInterrupt(x_39); +if (x_41 == 0) +{ +uint8_t x_42; +x_42 = l_Lean_Exception_isRuntime(x_39); +if (x_42 == 0) +{ +lean_object* x_43; +lean_free_object(x_31); +lean_inc(x_9); +x_43 = l_Lean_Elab_logException___at_Lean_Elab_Term_exceptionToSorry___spec__1(x_39, x_5, x_6, x_7, x_8, x_9, x_10, x_40); +if (lean_obj_tag(x_43) == 0) +{ +lean_object* x_44; size_t x_45; size_t x_46; +x_44 = lean_ctor_get(x_43, 1); +lean_inc(x_44); +lean_dec(x_43); +x_45 = 1; +x_46 = lean_usize_add(x_3, x_45); +x_3 = x_46; +x_11 = x_44; +goto _start; +} +else +{ +uint8_t x_48; +lean_dec(x_9); +lean_dec(x_5); lean_dec(x_4); -x_15 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkLevelNames___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_11); +x_48 = !lean_is_exclusive(x_43); +if (x_48 == 0) +{ +return x_43; +} +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; +} +} +} +else +{ lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_2); -lean_dec(x_1); -return x_15; +lean_dec(x_5); +lean_dec(x_4); +return x_31; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkLevelNames___boxed(lean_object* x_1, lean_object* x_2, lean_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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkLevelNames(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_7); +lean_dec(x_9); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -return x_9; +return x_31; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkTypeFor___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) { +else +{ +lean_object* x_52; lean_object* x_53; uint8_t x_54; +x_52 = lean_ctor_get(x_31, 0); +x_53 = lean_ctor_get(x_31, 1); +lean_inc(x_53); +lean_inc(x_52); +lean_dec(x_31); +x_54 = l_Lean_Exception_isInterrupt(x_52); +if (x_54 == 0) +{ +uint8_t x_55; +x_55 = l_Lean_Exception_isRuntime(x_52); +if (x_55 == 0) +{ +lean_object* x_56; +lean_inc(x_9); +x_56 = l_Lean_Elab_logException___at_Lean_Elab_Term_exceptionToSorry___spec__1(x_52, x_5, x_6, x_7, x_8, x_9, x_10, x_53); +if (lean_obj_tag(x_56) == 0) +{ +lean_object* x_57; size_t x_58; size_t x_59; +x_57 = lean_ctor_get(x_56, 1); +lean_inc(x_57); +lean_dec(x_56); +x_58 = 1; +x_59 = lean_usize_add(x_3, x_58); +x_3 = x_59; +x_11 = x_57; +goto _start; +} +else +{ +lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; +lean_dec(x_9); +lean_dec(x_5); +lean_dec(x_4); +x_61 = lean_ctor_get(x_56, 0); +lean_inc(x_61); +x_62 = lean_ctor_get(x_56, 1); +lean_inc(x_62); +if (lean_is_exclusive(x_56)) { + lean_ctor_release(x_56, 0); + lean_ctor_release(x_56, 1); + x_63 = x_56; +} else { + lean_dec_ref(x_56); + x_63 = lean_box(0); +} +if (lean_is_scalar(x_63)) { + x_64 = lean_alloc_ctor(1, 2, 0); +} else { + x_64 = x_63; +} +lean_ctor_set(x_64, 0, x_61); +lean_ctor_set(x_64, 1, x_62); +return x_64; +} +} +else +{ +lean_object* x_65; +lean_dec(x_9); +lean_dec(x_5); +lean_dec(x_4); +x_65 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_65, 0, x_52); +lean_ctor_set(x_65, 1, x_53); +return x_65; +} +} +else +{ +lean_object* x_66; +lean_dec(x_9); +lean_dec(x_5); +lean_dec(x_4); +x_66 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_66, 0, x_52); +lean_ctor_set(x_66, 1, x_53); +return x_66; +} +} +} +} +} +} +static lean_object* _init_l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__8___closed__1() { _start: { -uint8_t x_10; uint8_t x_11; uint8_t x_12; lean_object* x_13; -x_10 = 0; -x_11 = 1; -x_12 = 1; -x_13 = l_Lean_Meta_mkForallFVars(x_1, x_2, x_10, x_11, x_12, x_5, x_6, x_7, x_8, x_9); -return x_13; +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_array_mk(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkTypeFor(lean_object* x_1, lean_object* x_2, lean_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_elabAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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; 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 = lean_ctor_get(x_1, 2); -lean_inc(x_10); -x_11 = lean_ctor_get(x_1, 3); -lean_inc(x_11); -x_12 = lean_ctor_get(x_1, 4); -lean_inc(x_12); -lean_dec(x_1); -x_13 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkTypeFor___lambda__1___boxed), 9, 2); -lean_closure_set(x_13, 0, x_11); -lean_closure_set(x_13, 1, x_12); -x_14 = l_Lean_Meta_withLCtx___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__3___rarg(x_9, x_10, x_13, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -return x_14; +size_t x_9; size_t x_10; lean_object* x_11; lean_object* x_12; +x_9 = lean_array_size(x_1); +x_10 = 0; +x_11 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__8___closed__1; +x_12 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__16(x_1, x_9, x_10, x_11, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_12) == 0) +{ +uint8_t x_13; +x_13 = !lean_is_exclusive(x_12); +if (x_13 == 0) +{ +return x_12; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_12, 0); +x_15 = lean_ctor_get(x_12, 1); +lean_inc(x_15); +lean_inc(x_14); +lean_dec(x_12); +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_14); +lean_ctor_set(x_16, 1, x_15); +return x_16; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkTypeFor___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +else +{ +uint8_t x_17; +x_17 = !lean_is_exclusive(x_12); +if (x_17 == 0) +{ +return x_12; +} +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_EXPORT lean_object* l_Lean_Elab_elabDeclAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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: { -lean_object* x_10; -x_10 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkTypeFor___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -return x_10; +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_9 = lean_unsigned_to_nat(1u); +x_10 = l_Lean_Syntax_getArg(x_1, x_9); +x_11 = l_Lean_Syntax_getSepArgs(x_10); +lean_dec(x_10); +x_12 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__8(x_11, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_11); +return x_12; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___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_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__18(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; @@ -3559,954 +4648,1132 @@ return x_29; } } } -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___spec__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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) { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___spec__1___rarg___boxed), 8, 0); -return x_2; -} +uint8_t x_10; +x_10 = !lean_is_exclusive(x_7); +if (x_10 == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; +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_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__18(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_7); +return x_13; } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___rarg___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("unexpected inductive resulting type", 35, 35); -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; lean_object* x_23; lean_object* x_24; uint8_t x_25; lean_object* x_26; uint8_t x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_14 = lean_ctor_get(x_7, 0); +x_15 = lean_ctor_get(x_7, 1); +x_16 = lean_ctor_get(x_7, 2); +x_17 = lean_ctor_get(x_7, 3); +x_18 = lean_ctor_get(x_7, 4); +x_19 = lean_ctor_get(x_7, 5); +x_20 = lean_ctor_get(x_7, 6); +x_21 = lean_ctor_get(x_7, 7); +x_22 = lean_ctor_get(x_7, 8); +x_23 = lean_ctor_get(x_7, 9); +x_24 = lean_ctor_get(x_7, 10); +x_25 = lean_ctor_get_uint8(x_7, sizeof(void*)*12); +x_26 = lean_ctor_get(x_7, 11); +x_27 = lean_ctor_get_uint8(x_7, sizeof(void*)*12 + 1); +lean_inc(x_26); +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_inc(x_15); +lean_inc(x_14); +lean_dec(x_7); +x_28 = l_Lean_replaceRef(x_1, x_19); +lean_dec(x_19); +x_29 = lean_alloc_ctor(0, 12, 2); +lean_ctor_set(x_29, 0, x_14); +lean_ctor_set(x_29, 1, x_15); +lean_ctor_set(x_29, 2, x_16); +lean_ctor_set(x_29, 3, x_17); +lean_ctor_set(x_29, 4, x_18); +lean_ctor_set(x_29, 5, x_28); +lean_ctor_set(x_29, 6, x_20); +lean_ctor_set(x_29, 7, x_21); +lean_ctor_set(x_29, 8, x_22); +lean_ctor_set(x_29, 9, x_23); +lean_ctor_set(x_29, 10, x_24); +lean_ctor_set(x_29, 11, x_26); +lean_ctor_set_uint8(x_29, sizeof(void*)*12, x_25); +lean_ctor_set_uint8(x_29, sizeof(void*)*12 + 1, x_27); +x_30 = l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__18(x_2, x_3, x_4, x_5, x_6, x_29, x_8, x_9); +lean_dec(x_29); +return x_30; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___rarg___closed__2() { +} +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__21(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___rarg___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} +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_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_is_exclusive(x_12); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_14 = lean_ctor_get(x_12, 0); +x_15 = lean_ctor_get(x_12, 1); +x_16 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(x_14, x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_15); +lean_dec(x_2); +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_12, 1, x_18); +lean_ctor_set(x_12, 0, x_11); +lean_ctor_set_tag(x_16, 1); +lean_ctor_set(x_16, 0, x_12); +return x_16; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___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; -x_8 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___rarg___closed__2; -x_9 = l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___spec__1___rarg(x_8, x_1, x_2, x_3, x_4, x_5, x_6, x_7); -return x_9; +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_12, 1, x_19); +lean_ctor_set(x_12, 0, x_11); +x_21 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_21, 0, x_12); +lean_ctor_set(x_21, 1, x_20); +return x_21; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType(lean_object* x_1) { -_start: +else { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___rarg___boxed), 7, 0); -return x_2; +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_22 = lean_ctor_get(x_12, 0); +x_23 = lean_ctor_get(x_12, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_12); +x_24 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(x_22, x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_23); +lean_dec(x_2); +x_25 = lean_ctor_get(x_24, 0); +lean_inc(x_25); +x_26 = lean_ctor_get(x_24, 1); +lean_inc(x_26); +if (lean_is_exclusive(x_24)) { + lean_ctor_release(x_24, 0); + lean_ctor_release(x_24, 1); + x_27 = x_24; +} else { + lean_dec_ref(x_24); + x_27 = lean_box(0); +} +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_11); +lean_ctor_set(x_28, 1, x_25); +if (lean_is_scalar(x_27)) { + x_29 = lean_alloc_ctor(1, 2, 0); +} else { + x_29 = x_27; + lean_ctor_set_tag(x_29, 1); +} +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_26); +return x_29; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___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_Lean_throwErrorAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__20(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_9; -x_9 = l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +uint8_t x_10; +x_10 = !lean_is_exclusive(x_7); +if (x_10 == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; +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_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__21(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -return x_9; +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; 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; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_14 = lean_ctor_get(x_7, 0); +x_15 = lean_ctor_get(x_7, 1); +x_16 = lean_ctor_get(x_7, 2); +x_17 = lean_ctor_get(x_7, 3); +x_18 = lean_ctor_get(x_7, 4); +x_19 = lean_ctor_get(x_7, 5); +x_20 = lean_ctor_get(x_7, 6); +x_21 = lean_ctor_get(x_7, 7); +x_22 = lean_ctor_get(x_7, 8); +x_23 = lean_ctor_get(x_7, 9); +x_24 = lean_ctor_get(x_7, 10); +x_25 = lean_ctor_get_uint8(x_7, sizeof(void*)*12); +x_26 = lean_ctor_get(x_7, 11); +x_27 = lean_ctor_get_uint8(x_7, sizeof(void*)*12 + 1); +lean_inc(x_26); +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_inc(x_15); +lean_inc(x_14); +lean_dec(x_7); +x_28 = l_Lean_replaceRef(x_1, x_19); +lean_dec(x_19); +x_29 = lean_alloc_ctor(0, 12, 2); +lean_ctor_set(x_29, 0, x_14); +lean_ctor_set(x_29, 1, x_15); +lean_ctor_set(x_29, 2, x_16); +lean_ctor_set(x_29, 3, x_17); +lean_ctor_set(x_29, 4, x_18); +lean_ctor_set(x_29, 5, x_28); +lean_ctor_set(x_29, 6, x_20); +lean_ctor_set(x_29, 7, x_21); +lean_ctor_set(x_29, 8, x_22); +lean_ctor_set(x_29, 9, x_23); +lean_ctor_set(x_29, 10, x_24); +lean_ctor_set(x_29, 11, x_26); +lean_ctor_set_uint8(x_29, sizeof(void*)*12, x_25); +lean_ctor_set_uint8(x_29, sizeof(void*)*12 + 1, x_27); +x_30 = l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__21(x_2, x_3, x_4, x_5, x_6, x_29, x_8, x_9); +lean_dec(x_29); +return x_30; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___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_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__1() { _start: { -lean_object* x_8; -x_8 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_8; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("unexpected doc string", 21, 21); +return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_eqvFirstTypeResult___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +static lean_object* _init_l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__2() { _start: { -lean_object* x_9; -x_9 = l_Lean_Meta_isExprDefEq(x_3, x_1, x_4, x_5, x_6, x_7, x_8); -return x_9; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_eqvFirstTypeResult(lean_object* x_1, 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_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3() { _start: { -lean_object* x_8; uint8_t x_9; lean_object* x_10; -x_8 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_eqvFirstTypeResult___lambda__1___boxed), 8, 1); -lean_closure_set(x_8, 0, x_2); -x_9 = 0; -x_10 = l_Lean_Meta_forallTelescopeReducing___at_Lean_Meta_getParamNames___spec__2___rarg(x_1, x_8, x_9, x_3, x_4, x_5, x_6, x_7); -return x_10; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_45____closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_eqvFirstTypeResult___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_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_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_9; -x_9 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_eqvFirstTypeResult___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_object* x_9; lean_object* x_10; +x_9 = lean_unsigned_to_nat(1u); +x_10 = l_Lean_Syntax_getArg(x_1, x_9); +if (lean_obj_tag(x_10) == 2) +{ +uint8_t x_11; +lean_dec(x_6); lean_dec(x_2); -return x_9; +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_12 = lean_ctor_get(x_10, 1); +x_13 = lean_ctor_get(x_10, 0); +lean_dec(x_13); +x_14 = lean_string_utf8_byte_size(x_12); +x_15 = lean_unsigned_to_nat(2u); +x_16 = lean_nat_sub(x_14, x_15); +lean_dec(x_14); +x_17 = lean_unsigned_to_nat(0u); +x_18 = lean_string_utf8_extract(x_12, x_17, x_16); +lean_dec(x_16); +lean_dec(x_12); +lean_ctor_set_tag(x_10, 0); +lean_ctor_set(x_10, 1, x_8); +lean_ctor_set(x_10, 0, x_18); +return x_10; +} +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; +x_19 = lean_ctor_get(x_10, 1); +lean_inc(x_19); +lean_dec(x_10); +x_20 = lean_string_utf8_byte_size(x_19); +x_21 = lean_unsigned_to_nat(2u); +x_22 = lean_nat_sub(x_20, x_21); +lean_dec(x_20); +x_23 = lean_unsigned_to_nat(0u); +x_24 = lean_string_utf8_extract(x_19, x_23, x_22); +lean_dec(x_22); +lean_dec(x_19); +x_25 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_25, 0, x_24); +lean_ctor_set(x_25, 1, x_8); +return x_25; } } -LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___spec__1___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: +else { -lean_object* x_11; -x_11 = lean_apply_9(x_1, x_4, x_5, x_2, x_3, x_6, x_7, x_8, x_9, x_10); -return x_11; +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_26 = l_Lean_MessageData_ofSyntax(x_10); +x_27 = l_Lean_indentD(x_26); +x_28 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__2; +x_29 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_27); +x_30 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +x_31 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_31, 0, x_29); +lean_ctor_set(x_31, 1, x_30); +x_32 = l_Lean_throwErrorAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__20(x_1, x_31, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +return x_32; } } -LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___spec__1___rarg(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_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { -lean_object* x_11; lean_object* x_12; -x_11 = lean_alloc_closure((void*)(l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___spec__1___rarg___lambda__1), 10, 3); -lean_closure_set(x_11, 0, x_2); -lean_closure_set(x_11, 1, x_4); -lean_closure_set(x_11, 2, x_5); -x_12 = l___private_Lean_Meta_Basic_0__Lean_Meta_forallTelescopeReducingImp___rarg(x_1, x_11, x_3, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_12) == 0) +uint8_t x_15; uint8_t x_16; +x_15 = l_Lean_Syntax_isNone(x_1); +x_16 = l_Lean_Syntax_isNone(x_2); +if (x_15 == 0) { -uint8_t x_13; -x_13 = !lean_is_exclusive(x_12); -if (x_13 == 0) +if (x_16 == 0) { -return x_12; +uint8_t x_17; lean_object* x_18; lean_object* x_19; +x_17 = 1; +x_18 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_18, 0, x_3); +lean_ctor_set(x_18, 1, x_4); +lean_ctor_set(x_18, 2, x_7); +lean_ctor_set_uint8(x_18, sizeof(void*)*3, x_5); +lean_ctor_set_uint8(x_18, sizeof(void*)*3 + 1, x_17); +lean_ctor_set_uint8(x_18, sizeof(void*)*3 + 2, x_6); +lean_ctor_set_uint8(x_18, sizeof(void*)*3 + 3, x_17); +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set(x_19, 1, x_14); +return x_19; } else { -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; +uint8_t x_20; uint8_t x_21; lean_object* x_22; lean_object* x_23; +x_20 = 1; +x_21 = 0; +x_22 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_22, 0, x_3); +lean_ctor_set(x_22, 1, x_4); +lean_ctor_set(x_22, 2, x_7); +lean_ctor_set_uint8(x_22, sizeof(void*)*3, x_5); +lean_ctor_set_uint8(x_22, sizeof(void*)*3 + 1, x_20); +lean_ctor_set_uint8(x_22, sizeof(void*)*3 + 2, x_6); +lean_ctor_set_uint8(x_22, sizeof(void*)*3 + 3, x_21); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_14); +return x_23; } } else { -uint8_t x_17; -x_17 = !lean_is_exclusive(x_12); -if (x_17 == 0) +if (x_16 == 0) { -return x_12; +uint8_t x_24; uint8_t x_25; lean_object* x_26; lean_object* x_27; +x_24 = 0; +x_25 = 1; +x_26 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_26, 0, x_3); +lean_ctor_set(x_26, 1, x_4); +lean_ctor_set(x_26, 2, x_7); +lean_ctor_set_uint8(x_26, sizeof(void*)*3, x_5); +lean_ctor_set_uint8(x_26, sizeof(void*)*3 + 1, x_24); +lean_ctor_set_uint8(x_26, sizeof(void*)*3 + 2, x_6); +lean_ctor_set_uint8(x_26, sizeof(void*)*3 + 3, x_25); +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_14); +return x_27; } else { -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; +uint8_t x_28; lean_object* x_29; lean_object* x_30; +x_28 = 0; +x_29 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_29, 0, x_3); +lean_ctor_set(x_29, 1, x_4); +lean_ctor_set(x_29, 2, x_7); +lean_ctor_set_uint8(x_29, sizeof(void*)*3, x_5); +lean_ctor_set_uint8(x_29, sizeof(void*)*3 + 1, x_28); +lean_ctor_set_uint8(x_29, sizeof(void*)*3 + 2, x_6); +lean_ctor_set_uint8(x_29, sizeof(void*)*3 + 3, x_28); +x_30 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_30, 0, x_29); +lean_ctor_set(x_30, 1, x_14); +return x_30; } } } } -LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___spec__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, lean_object* x_6, uint8_t x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___spec__1___rarg___boxed), 10, 0); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeCompatible___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___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_15; +x_15 = l_Lean_Syntax_getOptional_x3f(x_6); +if (lean_obj_tag(x_15) == 0) { -lean_object* x_12; -x_12 = lean_apply_10(x_1, x_4, x_5, x_6, x_2, x_3, x_7, x_8, x_9, x_10, x_11); -return x_12; -} +lean_object* x_16; lean_object* x_17; +x_16 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__8___closed__1; +x_17 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__1(x_1, x_2, x_3, x_4, x_7, x_5, x_16, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_12); +lean_dec(x_8); +return x_17; } -LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeCompatible___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_12 = lean_alloc_closure((void*)(l_Lean_Meta_forallTelescopeCompatible___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___spec__2___lambda__1), 11, 3); -lean_closure_set(x_12, 0, x_4); -lean_closure_set(x_12, 1, x_5); -lean_closure_set(x_12, 2, x_6); -x_13 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__3___closed__1; -x_14 = l_Lean_Meta_forallTelescopeCompatibleAux___rarg(x_12, x_3, x_1, x_2, x_13, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_14) == 0) +else { -uint8_t x_15; -x_15 = !lean_is_exclusive(x_14); -if (x_15 == 0) +lean_object* x_18; lean_object* x_19; +x_18 = lean_ctor_get(x_15, 0); +lean_inc(x_18); +lean_dec(x_15); +lean_inc(x_12); +lean_inc(x_8); +x_19 = l_Lean_Elab_elabDeclAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__7(x_18, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_18); +if (lean_obj_tag(x_19) == 0) { -return x_14; +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_19, 1); +lean_inc(x_21); +lean_dec(x_19); +x_22 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__1(x_1, x_2, x_3, x_4, x_7, x_5, x_20, x_8, x_9, x_10, x_11, x_12, x_13, x_21); +lean_dec(x_12); +lean_dec(x_8); +return x_22; } else { -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_14, 0); -x_17 = lean_ctor_get(x_14, 1); -lean_inc(x_17); -lean_inc(x_16); -lean_dec(x_14); -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_16); -lean_ctor_set(x_18, 1, x_17); -return x_18; -} +uint8_t x_23; +lean_dec(x_12); +lean_dec(x_8); +lean_dec(x_4); +lean_dec(x_3); +x_23 = !lean_is_exclusive(x_19); +if (x_23 == 0) +{ +return x_19; } else { -uint8_t x_19; -x_19 = !lean_is_exclusive(x_14); -if (x_19 == 0) -{ -return x_14; +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_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 +} +} +} +} +static lean_object* _init_l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__1() { +_start: { -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_14, 0); -x_21 = lean_ctor_get(x_14, 1); -lean_inc(x_21); -lean_inc(x_20); -lean_dec(x_14); -x_22 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_22, 0, x_20); -lean_ctor_set(x_22, 1, x_21); -return x_22; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("private", 7, 7); +return x_1; } } +static lean_object* _init_l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; +x_2 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__1; +x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__7; +x_4 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__1; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__1___closed__1() { +static lean_object* _init_l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__3() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("resulting universe mismatch, given", 34, 34); +x_1 = lean_mk_string_unchecked("protected", 9, 9); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__1___closed__2() { +static lean_object* _init_l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__4() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__1___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; +x_2 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__1; +x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__7; +x_4 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__3; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__1___closed__3() { +static lean_object* _init_l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__5() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("\nexpected type", 14, 14); +x_1 = lean_mk_string_unchecked("unexpected visibility modifier", 30, 30); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__1___closed__4() { +static lean_object* _init_l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__6() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__1___closed__3; +x_1 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__5; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___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_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { -lean_object* x_11; -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -x_11 = l_Lean_Meta_whnfD(x_1, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_11) == 0) -{ -lean_object* x_12; -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); -if (lean_obj_tag(x_12) == 3) +lean_object* x_15; +x_15 = l_Lean_Syntax_getOptional_x3f(x_6); +if (lean_obj_tag(x_15) == 0) { -lean_object* x_13; lean_object* x_14; -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_12); -lean_inc(x_3); -x_14 = l_Lean_Meta_isExprDefEq(x_3, x_12, x_6, x_7, x_8, x_9, x_13); -if (lean_obj_tag(x_14) == 0) +uint8_t x_16; lean_object* x_17; +x_16 = 0; +x_17 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__2(x_1, x_2, x_3, x_7, x_4, x_5, x_16, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +return x_17; +} +else { -lean_object* x_15; uint8_t x_16; -x_15 = lean_ctor_get(x_14, 0); -lean_inc(x_15); -x_16 = lean_unbox(x_15); +lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_18 = lean_ctor_get(x_15, 0); +lean_inc(x_18); lean_dec(x_15); -if (x_16 == 0) +lean_inc(x_18); +x_19 = l_Lean_Syntax_getKind(x_18); +x_20 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__2; +x_21 = lean_name_eq(x_19, x_20); +if (x_21 == 0) { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_17 = lean_ctor_get(x_14, 1); -lean_inc(x_17); -lean_dec(x_14); -x_18 = l_Lean_indentExpr(x_12); -x_19 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__1___closed__2; -x_20 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_20, 0, x_19); -lean_ctor_set(x_20, 1, x_18); -x_21 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__1___closed__4; -x_22 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_22, 0, x_20); -lean_ctor_set(x_22, 1, x_21); -x_23 = l_Lean_indentExpr(x_3); -x_24 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_24, 0, x_22); -lean_ctor_set(x_24, 1, x_23); -x_25 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5; -x_26 = lean_alloc_ctor(7, 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_Term_throwErrorIfErrors___spec__1(x_26, x_4, x_5, x_6, x_7, x_8, x_9, x_17); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -return x_27; -} -else +lean_object* x_22; uint8_t x_23; +x_22 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__4; +x_23 = lean_name_eq(x_19, x_22); +lean_dec(x_19); +if (x_23 == 0) { -uint8_t x_28; -lean_dec(x_12); -lean_dec(x_9); -lean_dec(x_8); +lean_object* x_24; lean_object* x_25; uint8_t x_26; lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_4); lean_dec(x_3); -x_28 = !lean_is_exclusive(x_14); -if (x_28 == 0) +x_24 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__6; +x_25 = l_Lean_throwErrorAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__17(x_18, x_24, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_18); +x_26 = !lean_is_exclusive(x_25); +if (x_26 == 0) { -lean_object* x_29; lean_object* x_30; -x_29 = lean_ctor_get(x_14, 0); -lean_dec(x_29); -x_30 = lean_box(0); -lean_ctor_set(x_14, 0, x_30); -return x_14; +return x_25; } else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_31 = lean_ctor_get(x_14, 1); -lean_inc(x_31); -lean_dec(x_14); -x_32 = lean_box(0); -x_33 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_33, 0, x_32); -lean_ctor_set(x_33, 1, x_31); -return x_33; -} +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_25, 0); +x_28 = lean_ctor_get(x_25, 1); +lean_inc(x_28); +lean_inc(x_27); +lean_dec(x_25); +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_27); +lean_ctor_set(x_29, 1, x_28); +return x_29; } } else { -uint8_t x_34; -lean_dec(x_12); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_4); -lean_dec(x_3); -x_34 = !lean_is_exclusive(x_14); -if (x_34 == 0) -{ -return x_14; +uint8_t x_30; lean_object* x_31; +lean_dec(x_18); +x_30 = 1; +x_31 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__2(x_1, x_2, x_3, x_7, x_4, x_5, x_30, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +return x_31; +} } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_35 = lean_ctor_get(x_14, 0); -x_36 = lean_ctor_get(x_14, 1); -lean_inc(x_36); -lean_inc(x_35); -lean_dec(x_14); -x_37 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -return x_37; -} -} -} -else -{ -lean_object* x_38; lean_object* x_39; lean_object* x_40; -lean_dec(x_12); -lean_dec(x_3); -x_38 = lean_ctor_get(x_11, 1); -lean_inc(x_38); -lean_dec(x_11); -x_39 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___rarg___closed__2; -x_40 = l_Lean_throwError___at_Lean_Elab_Term_throwErrorIfErrors___spec__1(x_39, x_4, x_5, x_6, x_7, x_8, x_9, x_38); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -return x_40; -} -} -else -{ -uint8_t x_41; -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_4); -lean_dec(x_3); -x_41 = !lean_is_exclusive(x_11); -if (x_41 == 0) -{ -return x_11; -} -else -{ -lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_ctor_get(x_11, 0); -x_43 = lean_ctor_get(x_11, 1); -lean_inc(x_43); -lean_inc(x_42); -lean_dec(x_11); -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; +uint8_t x_32; lean_object* x_33; +lean_dec(x_19); +lean_dec(x_18); +x_32 = 2; +x_33 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__2(x_1, x_2, x_3, x_7, x_4, x_5, x_32, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +return x_33; } } } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___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) { +static lean_object* _init_l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__1() { _start: { -lean_object* x_11; uint8_t x_12; lean_object* x_13; -x_11 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__1___boxed), 10, 1); -lean_closure_set(x_11, 0, x_3); -x_12 = 0; -x_13 = l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___spec__1___rarg(x_1, x_11, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_13; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("partial", 7, 7); +return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___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) { +static lean_object* _init_l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__2() { _start: { -lean_object* x_11; uint8_t x_12; lean_object* x_13; -x_11 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__2___boxed), 10, 1); -lean_closure_set(x_11, 0, x_3); -x_12 = 0; -x_13 = l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___spec__1___rarg(x_2, x_11, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_13; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; +x_2 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__1; +x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__7; +x_4 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__1; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___closed__1() { +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__3___boxed), 10, 0); -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; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; lean_object* x_22; uint8_t x_23; +x_9 = lean_unsigned_to_nat(0u); +x_10 = l_Lean_Syntax_getArg(x_1, x_9); +x_11 = lean_unsigned_to_nat(1u); +x_12 = l_Lean_Syntax_getArg(x_1, x_11); +x_13 = lean_unsigned_to_nat(2u); +x_14 = l_Lean_Syntax_getArg(x_1, x_13); +x_15 = lean_unsigned_to_nat(3u); +x_16 = l_Lean_Syntax_getArg(x_1, x_15); +x_17 = lean_unsigned_to_nat(4u); +x_18 = l_Lean_Syntax_getArg(x_1, x_17); +x_19 = lean_unsigned_to_nat(5u); +x_20 = l_Lean_Syntax_getArg(x_1, x_19); +x_21 = l_Lean_Syntax_isNone(x_20); +x_22 = l_Lean_Syntax_getOptional_x3f(x_10); +lean_dec(x_10); +if (x_21 == 0) +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; uint8_t x_50; +x_47 = l_Lean_Syntax_getArg(x_20, x_9); +lean_dec(x_20); +x_48 = l_Lean_Syntax_getKind(x_47); +x_49 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__2; +x_50 = lean_name_eq(x_48, x_49); +lean_dec(x_48); +if (x_50 == 0) +{ +uint8_t x_51; +x_51 = 1; +x_23 = x_51; +goto block_46; } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___closed__2() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("invalid mutually inductive types, ", 34, 34); -return x_1; +uint8_t x_52; +x_52 = 0; +x_23 = x_52; +goto block_46; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___closed__3() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___closed__2; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} +uint8_t x_53; +lean_dec(x_20); +x_53 = 2; +x_23 = x_53; +goto block_46; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: +block_46: { -lean_object* x_11; lean_object* x_12; -x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___closed__1; -x_12 = l_Lean_Meta_forallTelescopeCompatible___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___spec__2(x_1, x_2, x_3, x_11, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_12) == 0) +if (lean_obj_tag(x_22) == 0) { -return x_12; +lean_object* x_24; lean_object* x_25; +x_24 = lean_box(0); +x_25 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3(x_16, x_18, x_1, x_23, x_12, x_14, x_24, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_14); +lean_dec(x_12); +lean_dec(x_18); +lean_dec(x_16); +return x_25; } else { -uint8_t x_13; -x_13 = !lean_is_exclusive(x_12); -if (x_13 == 0) -{ -lean_object* x_14; uint8_t x_15; -x_14 = lean_ctor_get(x_12, 0); -x_15 = l_Lean_Exception_isInterrupt(x_14); -if (x_15 == 0) -{ -uint8_t x_16; -x_16 = l_Lean_Exception_isRuntime(x_14); -if (x_16 == 0) -{ -if (lean_obj_tag(x_14) == 0) +uint8_t x_26; +x_26 = !lean_is_exclusive(x_22); +if (x_26 == 0) { -uint8_t x_17; -x_17 = !lean_is_exclusive(x_14); -if (x_17 == 0) +lean_object* x_27; lean_object* x_28; +x_27 = lean_ctor_get(x_22, 0); +lean_inc(x_6); +lean_inc(x_2); +x_28 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19(x_27, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_27); +if (lean_obj_tag(x_28) == 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); -x_19 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___closed__3; -x_20 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_20, 0, x_19); -lean_ctor_set(x_20, 1, x_18); -x_21 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5; -x_22 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_22, 0, x_20); -lean_ctor_set(x_22, 1, x_21); -lean_ctor_set(x_14, 1, x_22); -return x_12; +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_28, 0); +lean_inc(x_29); +x_30 = lean_ctor_get(x_28, 1); +lean_inc(x_30); +lean_dec(x_28); +lean_ctor_set(x_22, 0, x_29); +x_31 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3(x_16, x_18, x_1, x_23, x_12, x_14, x_22, x_2, x_3, x_4, x_5, x_6, x_7, x_30); +lean_dec(x_14); +lean_dec(x_12); +lean_dec(x_18); +lean_dec(x_16); +return x_31; } 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; -x_23 = lean_ctor_get(x_14, 0); -x_24 = lean_ctor_get(x_14, 1); -lean_inc(x_24); -lean_inc(x_23); +uint8_t x_32; +lean_free_object(x_22); +lean_dec(x_18); +lean_dec(x_16); lean_dec(x_14); -x_25 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___closed__3; -x_26 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_26, 1, x_24); -x_27 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5; -x_28 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_28, 0, x_26); -lean_ctor_set(x_28, 1, x_27); -x_29 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_29, 0, x_23); -lean_ctor_set(x_29, 1, x_28); -lean_ctor_set(x_12, 0, x_29); -return x_12; -} -} -else +lean_dec(x_12); +lean_dec(x_6); +lean_dec(x_2); +lean_dec(x_1); +x_32 = !lean_is_exclusive(x_28); +if (x_32 == 0) { -return x_12; -} +return x_28; } else { -return x_12; +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_28, 0); +x_34 = lean_ctor_get(x_28, 1); +lean_inc(x_34); +lean_inc(x_33); +lean_dec(x_28); +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +return x_35; +} } } else { -return x_12; -} +lean_object* x_36; lean_object* x_37; +x_36 = lean_ctor_get(x_22, 0); +lean_inc(x_36); +lean_dec(x_22); +lean_inc(x_6); +lean_inc(x_2); +x_37 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19(x_36, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_36); +if (lean_obj_tag(x_37) == 0) +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_38 = lean_ctor_get(x_37, 0); +lean_inc(x_38); +x_39 = lean_ctor_get(x_37, 1); +lean_inc(x_39); +lean_dec(x_37); +x_40 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_40, 0, x_38); +x_41 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3(x_16, x_18, x_1, x_23, x_12, x_14, x_40, x_2, x_3, x_4, x_5, x_6, x_7, x_39); +lean_dec(x_14); +lean_dec(x_12); +lean_dec(x_18); +lean_dec(x_16); +return x_41; } else { -lean_object* x_30; lean_object* x_31; uint8_t x_32; -x_30 = lean_ctor_get(x_12, 0); -x_31 = lean_ctor_get(x_12, 1); -lean_inc(x_31); -lean_inc(x_30); +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; +lean_dec(x_18); +lean_dec(x_16); +lean_dec(x_14); lean_dec(x_12); -x_32 = l_Lean_Exception_isInterrupt(x_30); -if (x_32 == 0) -{ -uint8_t x_33; -x_33 = l_Lean_Exception_isRuntime(x_30); -if (x_33 == 0) -{ -if (lean_obj_tag(x_30) == 0) -{ -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_34 = lean_ctor_get(x_30, 0); -lean_inc(x_34); -x_35 = lean_ctor_get(x_30, 1); -lean_inc(x_35); -if (lean_is_exclusive(x_30)) { - lean_ctor_release(x_30, 0); - lean_ctor_release(x_30, 1); - x_36 = x_30; +lean_dec(x_6); +lean_dec(x_2); +lean_dec(x_1); +x_42 = lean_ctor_get(x_37, 0); +lean_inc(x_42); +x_43 = lean_ctor_get(x_37, 1); +lean_inc(x_43); +if (lean_is_exclusive(x_37)) { + lean_ctor_release(x_37, 0); + lean_ctor_release(x_37, 1); + x_44 = x_37; } else { - lean_dec_ref(x_30); - x_36 = lean_box(0); + lean_dec_ref(x_37); + x_44 = lean_box(0); } -x_37 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___closed__3; -x_38 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_38, 0, x_37); -lean_ctor_set(x_38, 1, x_35); -x_39 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5; -x_40 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_40, 0, x_38); -lean_ctor_set(x_40, 1, x_39); -if (lean_is_scalar(x_36)) { - x_41 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_44)) { + x_45 = lean_alloc_ctor(1, 2, 0); } else { - x_41 = x_36; + x_45 = x_44; +} +lean_ctor_set(x_45, 0, x_42); +lean_ctor_set(x_45, 1, x_43); +return x_45; +} +} } -lean_ctor_set(x_41, 0, x_34); -lean_ctor_set(x_41, 1, x_40); -x_42 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_42, 0, x_41); -lean_ctor_set(x_42, 1, x_31); -return x_42; } -else -{ -lean_object* x_43; -x_43 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_43, 0, x_30); -lean_ctor_set(x_43, 1, x_31); -return x_43; } } +LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__22___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_10 = lean_ctor_get(x_1, 2); +x_11 = lean_array_get_size(x_10); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_nat_dec_eq(x_11, x_12); +lean_dec(x_11); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; +x_14 = l_Lean_Elab_Command_checkValidCtorModifier___rarg___lambda__1___closed__2; +x_15 = l_Lean_throwError___at_Lean_Elab_Term_throwErrorIfErrors___spec__1(x_14, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_15; +} else { -lean_object* x_44; -x_44 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_44, 0, x_30); -lean_ctor_set(x_44, 1, x_31); -return x_44; +lean_object* x_16; lean_object* x_17; +lean_dec(x_3); +x_16 = lean_box(0); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_16); +lean_ctor_set(x_17, 1, x_9); +return x_17; +} } } +LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__22___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +uint8_t x_10; +x_10 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 3); +if (x_10 == 0) +{ +lean_object* x_11; lean_object* x_12; +x_11 = lean_box(0); +x_12 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__22___lambda__1(x_1, x_11, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_12; +} else { -lean_object* x_45; -x_45 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_45, 0, x_30); -lean_ctor_set(x_45, 1, x_31); -return x_45; +lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_13 = l_Lean_Elab_Command_checkValidCtorModifier___rarg___lambda__2___closed__2; +x_14 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 0) +{ +return x_14; } +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_14, 0); +x_17 = lean_ctor_get(x_14, 1); +lean_inc(x_17); +lean_inc(x_16); +lean_dec(x_14); +x_18 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_18, 0, x_16); +lean_ctor_set(x_18, 1, x_17); +return x_18; } } } } -LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__22___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_11; lean_object* x_12; -x_11 = lean_unbox(x_3); -lean_dec(x_3); -x_12 = l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___spec__1___rarg(x_1, x_2, x_11, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +uint8_t x_10; +x_10 = l_Lean_Elab_Modifiers_isPartial(x_1); +if (x_10 == 0) +{ +lean_object* x_11; lean_object* x_12; +x_11 = lean_box(0); +x_12 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__22___lambda__2(x_1, x_11, x_3, x_4, x_5, x_6, x_7, x_8, x_9); return x_12; } +else +{ +lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_13 = l_Lean_Elab_Command_checkValidCtorModifier___rarg___lambda__3___closed__2; +x_14 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 0) +{ +return x_14; } -LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeCompatible___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: +else { -lean_object* x_12; -x_12 = l_Lean_Meta_forallTelescopeCompatible___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___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_3); -return x_12; +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_14, 0); +x_17 = lean_ctor_get(x_14, 1); +lean_inc(x_17); +lean_inc(x_16); +lean_dec(x_14); +x_18 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_18, 0, x_16); +lean_ctor_set(x_18, 1, x_17); +return x_18; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, 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_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___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_2); -return x_11; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__22(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_11; -x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___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_2); +uint8_t x_9; +x_9 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 1); +if (x_9 == 0) +{ +lean_object* x_10; lean_object* x_11; +x_10 = lean_box(0); +x_11 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__22___lambda__3(x_1, x_10, 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; uint8_t x_14; +x_12 = l_Lean_Elab_Command_checkValidCtorModifier___rarg___closed__2; +x_13 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_14 = !lean_is_exclusive(x_13); +if (x_14 == 0) +{ +return x_13; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: +else { -lean_object* x_11; -x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___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_1); -return x_11; +lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_15 = lean_ctor_get(x_13, 0); +x_16 = lean_ctor_get(x_13, 1); +lean_inc(x_16); +lean_inc(x_15); +lean_dec(x_13); +x_17 = lean_alloc_ctor(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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, 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_Inductive_0__Lean_Elab_Command_checkParamsAndResultType(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_Inductive_0__Lean_Elab_Command_checkHeader(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_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_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_11; -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); +lean_object* x_12; lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_1); -x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkTypeFor(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_11) == 0) +x_12 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__22(x_1, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_12) == 0) { -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; 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; uint8_t x_30; lean_object* x_31; uint8_t x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_13 = lean_ctor_get(x_12, 1); +lean_inc(x_13); +lean_dec(x_12); +x_14 = lean_unsigned_to_nat(3u); +x_15 = l_Lean_Syntax_getIdAt(x_2, x_14); +x_16 = l_Lean_Name_append(x_3, x_15); +x_17 = l_Lean_Syntax_getArg(x_2, x_14); +x_18 = lean_ctor_get_uint8(x_1, sizeof(void*)*3); +x_19 = lean_ctor_get(x_9, 0); +lean_inc(x_19); +x_20 = lean_ctor_get(x_9, 1); +lean_inc(x_20); +x_21 = lean_ctor_get(x_9, 2); +lean_inc(x_21); +x_22 = lean_ctor_get(x_9, 3); +lean_inc(x_22); +x_23 = lean_ctor_get(x_9, 4); +lean_inc(x_23); +x_24 = lean_ctor_get(x_9, 5); +lean_inc(x_24); +x_25 = lean_ctor_get(x_9, 6); +lean_inc(x_25); +x_26 = lean_ctor_get(x_9, 7); +lean_inc(x_26); +x_27 = lean_ctor_get(x_9, 8); +lean_inc(x_27); +x_28 = lean_ctor_get(x_9, 9); +lean_inc(x_28); +x_29 = lean_ctor_get(x_9, 10); +lean_inc(x_29); +x_30 = lean_ctor_get_uint8(x_9, sizeof(void*)*12); +x_31 = lean_ctor_get(x_9, 11); +lean_inc(x_31); +x_32 = lean_ctor_get_uint8(x_9, sizeof(void*)*12 + 1); +x_33 = l_Lean_replaceRef(x_17, x_24); +lean_dec(x_24); +x_34 = lean_alloc_ctor(0, 12, 2); +lean_ctor_set(x_34, 0, x_19); +lean_ctor_set(x_34, 1, x_20); +lean_ctor_set(x_34, 2, x_21); +lean_ctor_set(x_34, 3, x_22); +lean_ctor_set(x_34, 4, x_23); +lean_ctor_set(x_34, 5, x_33); +lean_ctor_set(x_34, 6, x_25); +lean_ctor_set(x_34, 7, x_26); +lean_ctor_set(x_34, 8, x_27); +lean_ctor_set(x_34, 9, x_28); +lean_ctor_set(x_34, 10, x_29); +lean_ctor_set(x_34, 11, x_31); +lean_ctor_set_uint8(x_34, sizeof(void*)*12, x_30); +lean_ctor_set_uint8(x_34, sizeof(void*)*12 + 1, x_32); +lean_inc(x_5); +x_35 = l_Lean_Elab_applyVisibility___at_Lean_Elab_Term_expandDeclId___spec__5(x_18, x_16, x_5, x_6, x_7, x_8, x_34, x_10, x_13); +lean_dec(x_34); +if (lean_obj_tag(x_35) == 0) { -uint8_t x_12; -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); +lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_36 = lean_ctor_get(x_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_unsigned_to_nat(4u); +x_39 = l_Lean_Syntax_getArg(x_2, x_38); +x_40 = l_Lean_Elab_expandOptDeclSig(x_39); +lean_dec(x_39); +x_41 = lean_ctor_get(x_40, 0); +lean_inc(x_41); +x_42 = lean_ctor_get(x_40, 1); +lean_inc(x_42); +lean_dec(x_40); +x_43 = lean_ctor_get(x_1, 1); +lean_inc(x_43); +lean_inc(x_5); +lean_inc(x_36); +x_44 = l_Lean_addDocString_x27___at_Lean_Elab_Term_expandDeclId___spec__8(x_36, x_43, x_5, x_6, x_7, x_8, x_9, x_10, x_37); +if (lean_obj_tag(x_44) == 0) +{ +lean_object* x_45; lean_object* x_46; uint8_t x_47; +x_45 = lean_ctor_get(x_44, 1); +lean_inc(x_45); +lean_dec(x_44); +lean_inc(x_36); +x_46 = l_Lean_Elab_addDeclarationRangesFromSyntax___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3(x_36, x_2, x_17, x_5, x_6, x_7, x_8, x_9, x_10, x_45); lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_1); -x_12 = !lean_is_exclusive(x_11); -if (x_12 == 0) +lean_dec(x_17); +x_47 = !lean_is_exclusive(x_46); +if (x_47 == 0) { -return x_11; +lean_object* x_48; lean_object* x_49; +x_48 = lean_ctor_get(x_46, 0); +lean_dec(x_48); +x_49 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_49, 0, x_2); +lean_ctor_set(x_49, 1, x_1); +lean_ctor_set(x_49, 2, x_36); +lean_ctor_set(x_49, 3, x_41); +lean_ctor_set(x_49, 4, x_42); +lean_ctor_set(x_46, 0, x_49); +return x_46; } 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_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 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_51, 0, x_2); +lean_ctor_set(x_51, 1, x_1); +lean_ctor_set(x_51, 2, x_36); +lean_ctor_set(x_51, 3, x_41); +lean_ctor_set(x_51, 4, x_42); +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_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; -x_16 = lean_ctor_get(x_11, 0); -lean_inc(x_16); -x_17 = lean_ctor_get(x_11, 1); -lean_inc(x_17); -lean_dec(x_11); -x_18 = lean_ctor_get(x_3, 0); -lean_inc(x_18); -lean_dec(x_3); -x_19 = lean_ctor_get(x_1, 0); -lean_inc(x_19); +uint8_t x_53; +lean_dec(x_42); +lean_dec(x_41); +lean_dec(x_36); +lean_dec(x_17); +lean_dec(x_9); +lean_dec(x_5); +lean_dec(x_2); lean_dec(x_1); -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); -lean_dec(x_19); -x_21 = !lean_is_exclusive(x_8); -if (x_21 == 0) -{ -lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_22 = lean_ctor_get(x_8, 5); -x_23 = l_Lean_replaceRef(x_20, x_22); -lean_dec(x_22); -lean_dec(x_20); -lean_ctor_set(x_8, 5, x_23); -lean_inc(x_18); -x_24 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType(x_16, x_18, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_17); -if (lean_obj_tag(x_24) == 0) -{ -uint8_t x_25; -x_25 = !lean_is_exclusive(x_24); -if (x_25 == 0) -{ -lean_object* x_26; -x_26 = lean_ctor_get(x_24, 0); -lean_dec(x_26); -lean_ctor_set(x_24, 0, x_18); -return x_24; -} -else -{ -lean_object* x_27; lean_object* x_28; -x_27 = lean_ctor_get(x_24, 1); -lean_inc(x_27); -lean_dec(x_24); -x_28 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_28, 0, x_18); -lean_ctor_set(x_28, 1, x_27); -return x_28; -} -} -else -{ -uint8_t x_29; -lean_dec(x_18); -x_29 = !lean_is_exclusive(x_24); -if (x_29 == 0) -{ -return x_24; -} -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; -} -} -} -else -{ -lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; lean_object* x_45; uint8_t x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_33 = lean_ctor_get(x_8, 0); -x_34 = lean_ctor_get(x_8, 1); -x_35 = lean_ctor_get(x_8, 2); -x_36 = lean_ctor_get(x_8, 3); -x_37 = lean_ctor_get(x_8, 4); -x_38 = lean_ctor_get(x_8, 5); -x_39 = lean_ctor_get(x_8, 6); -x_40 = lean_ctor_get(x_8, 7); -x_41 = lean_ctor_get(x_8, 8); -x_42 = lean_ctor_get(x_8, 9); -x_43 = lean_ctor_get(x_8, 10); -x_44 = lean_ctor_get_uint8(x_8, sizeof(void*)*12); -x_45 = lean_ctor_get(x_8, 11); -x_46 = lean_ctor_get_uint8(x_8, sizeof(void*)*12 + 1); -lean_inc(x_45); -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_dec(x_8); -x_47 = l_Lean_replaceRef(x_20, x_38); -lean_dec(x_38); -lean_dec(x_20); -x_48 = lean_alloc_ctor(0, 12, 2); -lean_ctor_set(x_48, 0, x_33); -lean_ctor_set(x_48, 1, x_34); -lean_ctor_set(x_48, 2, x_35); -lean_ctor_set(x_48, 3, x_36); -lean_ctor_set(x_48, 4, x_37); -lean_ctor_set(x_48, 5, x_47); -lean_ctor_set(x_48, 6, x_39); -lean_ctor_set(x_48, 7, x_40); -lean_ctor_set(x_48, 8, x_41); -lean_ctor_set(x_48, 9, x_42); -lean_ctor_set(x_48, 10, x_43); -lean_ctor_set(x_48, 11, x_45); -lean_ctor_set_uint8(x_48, sizeof(void*)*12, x_44); -lean_ctor_set_uint8(x_48, sizeof(void*)*12 + 1, x_46); -lean_inc(x_18); -x_49 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType(x_16, x_18, x_2, x_4, x_5, x_6, x_7, x_48, x_9, x_17); -if (lean_obj_tag(x_49) == 0) +x_53 = !lean_is_exclusive(x_44); +if (x_53 == 0) { -lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_50 = lean_ctor_get(x_49, 1); -lean_inc(x_50); -if (lean_is_exclusive(x_49)) { - lean_ctor_release(x_49, 0); - lean_ctor_release(x_49, 1); - x_51 = x_49; -} else { - lean_dec_ref(x_49); - x_51 = lean_box(0); -} -if (lean_is_scalar(x_51)) { - x_52 = lean_alloc_ctor(0, 2, 0); -} else { - x_52 = x_51; -} -lean_ctor_set(x_52, 0, x_18); -lean_ctor_set(x_52, 1, x_50); -return x_52; +return x_44; } else { -lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; -lean_dec(x_18); -x_53 = lean_ctor_get(x_49, 0); -lean_inc(x_53); -x_54 = lean_ctor_get(x_49, 1); +lean_object* x_54; lean_object* x_55; lean_object* x_56; +x_54 = lean_ctor_get(x_44, 0); +x_55 = lean_ctor_get(x_44, 1); +lean_inc(x_55); lean_inc(x_54); -if (lean_is_exclusive(x_49)) { - lean_ctor_release(x_49, 0); - lean_ctor_release(x_49, 1); - x_55 = x_49; -} else { - lean_dec_ref(x_49); - x_55 = lean_box(0); -} -if (lean_is_scalar(x_55)) { - x_56 = lean_alloc_ctor(1, 2, 0); -} else { - x_56 = x_55; -} -lean_ctor_set(x_56, 0, x_53); -lean_ctor_set(x_56, 1, x_54); +lean_dec(x_44); +x_56 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_56, 0, x_54); +lean_ctor_set(x_56, 1, x_55); return x_56; } } } -} else { uint8_t x_57; +lean_dec(x_17); lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); +lean_dec(x_2); lean_dec(x_1); -x_57 = !lean_is_exclusive(x_11); +x_57 = !lean_is_exclusive(x_35); if (x_57 == 0) { -return x_11; +return x_35; } else { lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_58 = lean_ctor_get(x_11, 0); -x_59 = lean_ctor_get(x_11, 1); +x_58 = lean_ctor_get(x_35, 0); +x_59 = lean_ctor_get(x_35, 1); lean_inc(x_59); lean_inc(x_58); -lean_dec(x_11); +lean_dec(x_35); x_60 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_60, 0, x_58); lean_ctor_set(x_60, 1, x_59); @@ -4514,941 +5781,1141 @@ return x_60; } } } +else +{ +uint8_t x_61; +lean_dec(x_9); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_61 = !lean_is_exclusive(x_12); +if (x_61 == 0) +{ +return x_12; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkHeader___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +else +{ +lean_object* x_62; lean_object* x_63; lean_object* x_64; +x_62 = lean_ctor_get(x_12, 0); +x_63 = lean_ctor_get(x_12, 1); +lean_inc(x_63); +lean_inc(x_62); +lean_dec(x_12); +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; +} +} +} +} +static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__2___closed__1() { _start: { -lean_object* x_11; -x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkHeader(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_2); -return x_11; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("invalid 'protected' constructor in a 'private' inductive datatype", 65, 65); +return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkHeaders(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, 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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__2___closed__2() { _start: { -lean_object* x_12; uint8_t x_13; -x_12 = lean_array_get_size(x_1); -x_13 = lean_nat_dec_lt(x_3, x_12); -lean_dec(x_12); +lean_object* x_1; lean_object* x_2; +x_1 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__2___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___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; +x_13 = l_Lean_Elab_Modifiers_isProtected(x_1); if (x_13 == 0) { lean_object* x_14; lean_object* x_15; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); x_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_11); +x_15 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__1(x_1, x_2, x_3, x_14, x_6, x_7, x_8, x_9, x_10, x_11, x_12); return x_15; } else { -lean_object* x_16; lean_object* x_17; -x_16 = lean_array_fget(x_1, 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_5); -x_17 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkHeader(x_16, x_2, 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_16; +x_16 = l_Lean_Elab_Modifiers_isPrivate(x_4); +if (x_16 == 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_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_unsigned_to_nat(1u); -x_21 = lean_nat_add(x_3, x_20); -lean_dec(x_3); -x_22 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_22, 0, x_18); -x_3 = x_21; -x_4 = x_22; -x_11 = x_19; -goto _start; +lean_object* x_17; lean_object* x_18; +x_17 = lean_box(0); +x_18 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__1(x_1, x_2, x_3, x_17, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +return x_18; } 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); +lean_object* x_19; lean_object* x_20; uint8_t x_21; lean_dec(x_3); -x_24 = !lean_is_exclusive(x_17); -if (x_24 == 0) +lean_dec(x_2); +lean_dec(x_1); +x_19 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__2___closed__2; +x_20 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_19, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_10); +x_21 = !lean_is_exclusive(x_20); +if (x_21 == 0) { -return x_17; +return x_20; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_17, 0); -x_26 = lean_ctor_get(x_17, 1); -lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_17); -x_27 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_26); -return x_27; +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_20, 0); +x_23 = lean_ctor_get(x_20, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_20); +x_24 = lean_alloc_ctor(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_Inductive_0__Lean_Elab_Command_checkHeaders___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, 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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__3___closed__1() { _start: { -lean_object* x_12; -x_12 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkHeaders(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_2); -lean_dec(x_1); -return x_12; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("invalid 'private' constructor in a 'private' inductive datatype", 63, 63); +return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeader___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) { +static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__3___closed__2() { _start: { -lean_object* x_10; -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_1); -lean_ctor_set(x_10, 1, x_9); -return x_10; +lean_object* x_1; lean_object* x_2; +x_1 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__3___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeader(lean_object* x_1, lean_object* x_2, lean_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_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_9 = lean_unsigned_to_nat(0u); -x_10 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__3___closed__1; -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_2); -x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux(x_1, x_9, x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_11) == 0) +uint8_t x_13; +x_13 = l_Lean_Elab_Modifiers_isPrivate(x_4); +if (x_13 == 0) { -uint8_t x_12; -x_12 = !lean_is_exclusive(x_11); -if (x_12 == 0) +lean_object* x_14; lean_object* x_15; +x_14 = lean_box(0); +x_15 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__2(x_4, x_1, x_2, x_3, x_14, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +return x_15; +} +else { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; -x_13 = lean_ctor_get(x_11, 0); -x_14 = lean_ctor_get(x_11, 1); -x_15 = lean_array_get_size(x_13); -x_16 = lean_unsigned_to_nat(1u); -x_17 = lean_nat_dec_lt(x_16, x_15); -lean_dec(x_15); -if (x_17 == 0) +uint8_t x_16; +x_16 = l_Lean_Elab_Modifiers_isPrivate(x_3); +if (x_16 == 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); -return x_11; +lean_object* x_17; lean_object* x_18; +x_17 = lean_box(0); +x_18 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__2(x_4, x_1, x_2, x_3, x_17, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +return x_18; } else { -lean_object* x_18; -lean_free_object(x_11); -lean_inc(x_6); -lean_inc(x_2); -x_18 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe(x_13, x_2, x_3, x_4, x_5, x_6, x_7, x_14); -if (lean_obj_tag(x_18) == 0) +lean_object* x_19; lean_object* x_20; uint8_t x_21; +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_19 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__3___closed__2; +x_20 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_19, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_10); +x_21 = !lean_is_exclusive(x_20); +if (x_21 == 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); -lean_inc(x_6); -lean_inc(x_2); -x_20 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams(x_13, x_2, x_3, x_4, x_5, x_6, x_7, x_19); -if (lean_obj_tag(x_20) == 0) +return x_20; +} +else { -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_20, 1); +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_20, 0); +x_23 = lean_ctor_get(x_20, 1); +lean_inc(x_23); lean_inc(x_22); lean_dec(x_20); -x_23 = lean_box(0); -x_24 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkHeaders(x_13, x_21, x_9, x_23, x_2, x_3, x_4, x_5, x_6, x_7, x_22); -lean_dec(x_21); -if (lean_obj_tag(x_24) == 0) -{ -uint8_t x_25; -x_25 = !lean_is_exclusive(x_24); -if (x_25 == 0) -{ -lean_object* x_26; -x_26 = lean_ctor_get(x_24, 0); -lean_dec(x_26); -lean_ctor_set(x_24, 0, x_13); +x_24 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); return x_24; } -else -{ -lean_object* x_27; lean_object* x_28; -x_27 = lean_ctor_get(x_24, 1); -lean_inc(x_27); -lean_dec(x_24); -x_28 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_28, 0, x_13); -lean_ctor_set(x_28, 1, x_27); -return x_28; } } -else +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___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_29; -lean_dec(x_13); -x_29 = !lean_is_exclusive(x_24); -if (x_29 == 0) +uint8_t x_12; +x_12 = !lean_is_exclusive(x_3); +if (x_12 == 0) { -return x_24; +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_3, 1); +lean_dec(x_13); +x_14 = l_Lean_TSyntax_getDocString(x_1); +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_3, 1, x_15); +x_16 = lean_box(0); +x_17 = lean_apply_9(x_2, x_3, x_16, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_17; } 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_18; uint8_t x_19; uint8_t x_20; uint8_t 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; +x_18 = lean_ctor_get(x_3, 0); +x_19 = lean_ctor_get_uint8(x_3, sizeof(void*)*3); +x_20 = lean_ctor_get_uint8(x_3, sizeof(void*)*3 + 1); +x_21 = lean_ctor_get_uint8(x_3, sizeof(void*)*3 + 2); +x_22 = lean_ctor_get_uint8(x_3, sizeof(void*)*3 + 3); +x_23 = lean_ctor_get(x_3, 2); +lean_inc(x_23); +lean_inc(x_18); +lean_dec(x_3); +x_24 = l_Lean_TSyntax_getDocString(x_1); +x_25 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_25, 0, x_24); +x_26 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_26, 0, x_18); +lean_ctor_set(x_26, 1, x_25); +lean_ctor_set(x_26, 2, x_23); +lean_ctor_set_uint8(x_26, sizeof(void*)*3, x_19); +lean_ctor_set_uint8(x_26, sizeof(void*)*3 + 1, x_20); +lean_ctor_set_uint8(x_26, sizeof(void*)*3 + 2, x_21); +lean_ctor_set_uint8(x_26, sizeof(void*)*3 + 3, x_22); +x_27 = lean_box(0); +x_28 = lean_apply_9(x_2, x_26, x_27, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_28; } } } -else +static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___closed__1() { +_start: { -uint8_t x_33; -lean_dec(x_13); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_33 = !lean_is_exclusive(x_20); -if (x_33 == 0) +lean_object* x_1; +x_1 = lean_mk_string_unchecked("duplicate doc string", 20, 20); +return x_1; +} +} +static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___closed__2() { +_start: { -return x_20; +lean_object* x_1; lean_object* x_2; +x_1 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___closed__1; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; } -else +} +static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___closed__3() { +_start: { -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_20, 0); -x_35 = lean_ctor_get(x_20, 1); -lean_inc(x_35); -lean_inc(x_34); -lean_dec(x_20); -x_36 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_36, 0, x_34); -lean_ctor_set(x_36, 1, x_35); -return x_36; -} +lean_object* x_1; lean_object* x_2; +x_1 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___closed__2; +x_2 = l_Lean_MessageData_ofFormat(x_1); +return x_2; } } -else +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23(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_37; -lean_dec(x_13); +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_9); +lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); lean_dec(x_2); -x_37 = !lean_is_exclusive(x_18); -if (x_37 == 0) -{ -return x_18; +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_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_18, 0); -x_39 = lean_ctor_get(x_18, 1); -lean_inc(x_39); +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; lean_object* x_32; uint8_t x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; +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); +x_18 = lean_unsigned_to_nat(2u); +x_19 = l_Lean_Syntax_getArg(x_15, x_18); +x_20 = lean_ctor_get(x_10, 0); +x_21 = lean_ctor_get(x_10, 1); +x_22 = lean_ctor_get(x_10, 2); +x_23 = lean_ctor_get(x_10, 3); +x_24 = lean_ctor_get(x_10, 4); +x_25 = lean_ctor_get(x_10, 5); +x_26 = lean_ctor_get(x_10, 6); +x_27 = lean_ctor_get(x_10, 7); +x_28 = lean_ctor_get(x_10, 8); +x_29 = lean_ctor_get(x_10, 9); +x_30 = lean_ctor_get(x_10, 10); +x_31 = lean_ctor_get_uint8(x_10, sizeof(void*)*12); +x_32 = lean_ctor_get(x_10, 11); +x_33 = lean_ctor_get_uint8(x_10, sizeof(void*)*12 + 1); +x_34 = l_Lean_replaceRef(x_15, x_25); +lean_inc(x_32); +lean_inc(x_30); +lean_inc(x_29); +lean_inc(x_28); +lean_inc(x_27); +lean_inc(x_26); +lean_inc(x_24); +lean_inc(x_23); +lean_inc(x_22); +lean_inc(x_21); +lean_inc(x_20); +x_35 = lean_alloc_ctor(0, 12, 2); +lean_ctor_set(x_35, 0, x_20); +lean_ctor_set(x_35, 1, x_21); +lean_ctor_set(x_35, 2, x_22); +lean_ctor_set(x_35, 3, x_23); +lean_ctor_set(x_35, 4, x_24); +lean_ctor_set(x_35, 5, x_34); +lean_ctor_set(x_35, 6, x_26); +lean_ctor_set(x_35, 7, x_27); +lean_ctor_set(x_35, 8, x_28); +lean_ctor_set(x_35, 9, x_29); +lean_ctor_set(x_35, 10, x_30); +lean_ctor_set(x_35, 11, x_32); +lean_ctor_set_uint8(x_35, sizeof(void*)*12, x_31); +lean_ctor_set_uint8(x_35, sizeof(void*)*12 + 1, x_33); +lean_inc(x_35); +lean_inc(x_6); +x_36 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6(x_19, x_6, x_7, x_8, x_9, x_35, x_11, x_12); +if (lean_obj_tag(x_36) == 0) +{ +lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_37 = lean_ctor_get(x_36, 0); +lean_inc(x_37); +x_38 = lean_ctor_get(x_36, 1); lean_inc(x_38); -lean_dec(x_18); -x_40 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_40, 0, x_38); -lean_ctor_set(x_40, 1, x_39); -return x_40; -} -} -} +lean_dec(x_36); +lean_inc(x_1); +lean_inc(x_2); +lean_inc(x_15); +x_39 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__3___boxed), 12, 3); +lean_closure_set(x_39, 0, x_15); +lean_closure_set(x_39, 1, x_2); +lean_closure_set(x_39, 2, x_1); +x_40 = l_Lean_Syntax_getArg(x_15, x_16); +x_41 = l_Lean_Syntax_getOptional_x3f(x_40); +lean_dec(x_40); +if (lean_obj_tag(x_41) == 0) +{ +lean_object* x_42; lean_object* x_43; +lean_dec(x_39); +x_42 = lean_box(0); +lean_inc(x_6); +lean_inc(x_2); +x_43 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__3(x_15, x_2, x_1, x_37, x_42, x_6, x_7, x_8, x_9, x_35, x_11, x_38); +if (lean_obj_tag(x_43) == 0) +{ +lean_object* x_44; lean_object* x_45; size_t x_46; size_t x_47; lean_object* x_48; +x_44 = lean_ctor_get(x_43, 0); +lean_inc(x_44); +x_45 = lean_ctor_get(x_43, 1); +lean_inc(x_45); +lean_dec(x_43); +x_46 = 1; +x_47 = lean_usize_add(x_4, x_46); +x_48 = lean_array_uset(x_17, x_4, x_44); +x_4 = x_47; +x_5 = x_48; +x_12 = x_45; +goto _start; } 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_11, 0); -x_42 = lean_ctor_get(x_11, 1); -lean_inc(x_42); -lean_inc(x_41); +uint8_t x_50; +lean_dec(x_17); lean_dec(x_11); -x_43 = lean_array_get_size(x_41); -x_44 = lean_unsigned_to_nat(1u); -x_45 = lean_nat_dec_lt(x_44, x_43); -lean_dec(x_43); -if (x_45 == 0) -{ -lean_object* x_46; +lean_dec(x_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_46 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_46, 0, x_41); -lean_ctor_set(x_46, 1, x_42); -return x_46; +lean_dec(x_1); +x_50 = !lean_is_exclusive(x_43); +if (x_50 == 0) +{ +return x_43; } else { -lean_object* x_47; -lean_inc(x_6); -lean_inc(x_2); -x_47 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe(x_41, x_2, x_3, x_4, x_5, x_6, x_7, x_42); -if (lean_obj_tag(x_47) == 0) -{ -lean_object* x_48; lean_object* x_49; -x_48 = lean_ctor_get(x_47, 1); -lean_inc(x_48); -lean_dec(x_47); -lean_inc(x_6); -lean_inc(x_2); -x_49 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams(x_41, x_2, x_3, x_4, x_5, x_6, x_7, x_48); -if (lean_obj_tag(x_49) == 0) -{ -lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; -x_50 = lean_ctor_get(x_49, 0); -lean_inc(x_50); -x_51 = lean_ctor_get(x_49, 1); +lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_51 = lean_ctor_get(x_43, 0); +x_52 = lean_ctor_get(x_43, 1); +lean_inc(x_52); lean_inc(x_51); -lean_dec(x_49); -x_52 = lean_box(0); -x_53 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkHeaders(x_41, x_50, x_9, x_52, x_2, x_3, x_4, x_5, x_6, x_7, x_51); -lean_dec(x_50); -if (lean_obj_tag(x_53) == 0) -{ -lean_object* x_54; lean_object* x_55; lean_object* x_56; -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_53); - x_55 = lean_box(0); +lean_dec(x_43); +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; } -if (lean_is_scalar(x_55)) { - x_56 = lean_alloc_ctor(0, 2, 0); -} else { - x_56 = x_55; } -lean_ctor_set(x_56, 0, x_41); -lean_ctor_set(x_56, 1, x_54); -return x_56; } else { -lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; +lean_object* x_54; +lean_dec(x_15); +x_54 = lean_ctor_get(x_37, 1); +lean_inc(x_54); +if (lean_obj_tag(x_54) == 0) +{ +lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_55 = lean_ctor_get(x_41, 0); +lean_inc(x_55); lean_dec(x_41); -x_57 = lean_ctor_get(x_53, 0); -lean_inc(x_57); -x_58 = lean_ctor_get(x_53, 1); +x_56 = lean_box(0); +lean_inc(x_11); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +x_57 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__4(x_55, x_39, x_37, x_56, x_6, x_7, x_8, x_9, x_35, x_11, x_38); +lean_dec(x_55); +if (lean_obj_tag(x_57) == 0) +{ +lean_object* x_58; lean_object* x_59; size_t x_60; size_t x_61; lean_object* x_62; +x_58 = lean_ctor_get(x_57, 0); lean_inc(x_58); -if (lean_is_exclusive(x_53)) { - lean_ctor_release(x_53, 0); - lean_ctor_release(x_53, 1); - x_59 = x_53; -} else { - lean_dec_ref(x_53); - x_59 = lean_box(0); -} -if (lean_is_scalar(x_59)) { - x_60 = lean_alloc_ctor(1, 2, 0); -} else { - x_60 = x_59; -} -lean_ctor_set(x_60, 0, x_57); -lean_ctor_set(x_60, 1, x_58); -return x_60; -} +x_59 = lean_ctor_get(x_57, 1); +lean_inc(x_59); +lean_dec(x_57); +x_60 = 1; +x_61 = lean_usize_add(x_4, x_60); +x_62 = lean_array_uset(x_17, x_4, x_58); +x_4 = x_61; +x_5 = x_62; +x_12 = x_59; +goto _start; } else { -lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; -lean_dec(x_41); +uint8_t x_64; +lean_dec(x_17); +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); -lean_dec(x_3); lean_dec(x_2); -x_61 = lean_ctor_get(x_49, 0); -lean_inc(x_61); -x_62 = lean_ctor_get(x_49, 1); -lean_inc(x_62); -if (lean_is_exclusive(x_49)) { - lean_ctor_release(x_49, 0); - lean_ctor_release(x_49, 1); - x_63 = x_49; -} else { - lean_dec_ref(x_49); - x_63 = lean_box(0); +lean_dec(x_1); +x_64 = !lean_is_exclusive(x_57); +if (x_64 == 0) +{ +return x_57; } -if (lean_is_scalar(x_63)) { - x_64 = lean_alloc_ctor(1, 2, 0); -} else { - x_64 = x_63; +else +{ +lean_object* x_65; lean_object* x_66; lean_object* x_67; +x_65 = lean_ctor_get(x_57, 0); +x_66 = lean_ctor_get(x_57, 1); +lean_inc(x_66); +lean_inc(x_65); +lean_dec(x_57); +x_67 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_67, 0, x_65); +lean_ctor_set(x_67, 1, x_66); +return x_67; } -lean_ctor_set(x_64, 0, x_61); -lean_ctor_set(x_64, 1, x_62); -return x_64; } } else { -lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; +lean_object* x_68; lean_object* x_69; uint8_t x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; +lean_dec(x_54); +x_68 = lean_ctor_get(x_41, 0); +lean_inc(x_68); lean_dec(x_41); +x_69 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___closed__3; +x_70 = 2; +lean_inc(x_35); +x_71 = l_Lean_logAt___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__2(x_68, x_69, x_70, x_6, x_7, x_8, x_9, x_35, x_11, x_38); +x_72 = lean_ctor_get(x_71, 0); +lean_inc(x_72); +x_73 = lean_ctor_get(x_71, 1); +lean_inc(x_73); +lean_dec(x_71); +lean_inc(x_11); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +x_74 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__4(x_68, x_39, x_37, x_72, x_6, x_7, x_8, x_9, x_35, x_11, x_73); +lean_dec(x_72); +lean_dec(x_68); +if (lean_obj_tag(x_74) == 0) +{ +lean_object* x_75; lean_object* x_76; size_t x_77; size_t x_78; lean_object* x_79; +x_75 = lean_ctor_get(x_74, 0); +lean_inc(x_75); +x_76 = lean_ctor_get(x_74, 1); +lean_inc(x_76); +lean_dec(x_74); +x_77 = 1; +x_78 = lean_usize_add(x_4, x_77); +x_79 = lean_array_uset(x_17, x_4, x_75); +x_4 = x_78; +x_5 = x_79; +x_12 = x_76; +goto _start; +} +else +{ +uint8_t x_81; +lean_dec(x_17); +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); -lean_dec(x_3); lean_dec(x_2); -x_65 = lean_ctor_get(x_47, 0); -lean_inc(x_65); -x_66 = lean_ctor_get(x_47, 1); -lean_inc(x_66); -if (lean_is_exclusive(x_47)) { - lean_ctor_release(x_47, 0); - lean_ctor_release(x_47, 1); - x_67 = x_47; -} else { - lean_dec_ref(x_47); - x_67 = lean_box(0); +lean_dec(x_1); +x_81 = !lean_is_exclusive(x_74); +if (x_81 == 0) +{ +return x_74; } -if (lean_is_scalar(x_67)) { - x_68 = lean_alloc_ctor(1, 2, 0); -} else { - x_68 = x_67; +else +{ +lean_object* x_82; lean_object* x_83; lean_object* x_84; +x_82 = lean_ctor_get(x_74, 0); +x_83 = lean_ctor_get(x_74, 1); +lean_inc(x_83); +lean_inc(x_82); +lean_dec(x_74); +x_84 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_84, 0, x_82); +lean_ctor_set(x_84, 1, x_83); +return x_84; } -lean_ctor_set(x_68, 0, x_65); -lean_ctor_set(x_68, 1, x_66); -return x_68; } } } } else { -uint8_t x_69; +uint8_t x_85; +lean_dec(x_35); +lean_dec(x_17); +lean_dec(x_15); +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); -lean_dec(x_3); lean_dec(x_2); -x_69 = !lean_is_exclusive(x_11); -if (x_69 == 0) +lean_dec(x_1); +x_85 = !lean_is_exclusive(x_36); +if (x_85 == 0) { -return x_11; +return x_36; } else { -lean_object* x_70; lean_object* x_71; lean_object* x_72; -x_70 = lean_ctor_get(x_11, 0); -x_71 = lean_ctor_get(x_11, 1); -lean_inc(x_71); -lean_inc(x_70); -lean_dec(x_11); -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_86; lean_object* x_87; lean_object* x_88; +x_86 = lean_ctor_get(x_36, 0); +x_87 = lean_ctor_get(x_36, 1); +lean_inc(x_87); +lean_inc(x_86); +lean_dec(x_36); +x_88 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_88, 0, x_86); +lean_ctor_set(x_88, 1, x_87); +return x_88; } } } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeader___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__24(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: { -lean_object* x_10; -x_10 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeader___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_10; +uint8_t x_11; +x_11 = lean_usize_dec_lt(x_2, x_1); +if (x_11 == 0) +{ +lean_object* x_12; +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; 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; size_t x_26; lean_object* x_27; +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 = l_Lean_Syntax_getArg(x_13, x_14); +x_17 = lean_unsigned_to_nat(1u); +x_18 = l_Lean_Syntax_getArg(x_13, x_17); +x_19 = l_Lean_Syntax_getId(x_18); +lean_dec(x_18); +x_20 = lean_unsigned_to_nat(3u); +x_21 = l_Lean_Syntax_getArg(x_13, x_20); +x_22 = lean_unsigned_to_nat(4u); +x_23 = l_Lean_Syntax_getArg(x_13, x_22); +x_24 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_24, 0, x_13); +lean_ctor_set(x_24, 1, x_16); +lean_ctor_set(x_24, 2, x_19); +lean_ctor_set(x_24, 3, x_21); +lean_ctor_set(x_24, 4, x_23); +x_25 = 1; +x_26 = lean_usize_add(x_2, x_25); +x_27 = lean_array_uset(x_15, x_2, x_24); +x_2 = x_26; +x_3 = x_27; +goto _start; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls_loop___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +} +static lean_object* _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__1() { _start: { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_14 = lean_unsigned_to_nat(1u); -x_15 = lean_nat_add(x_1, x_14); -x_16 = lean_array_push(x_2, x_6); -x_17 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls_loop___rarg(x_3, x_4, x_5, x_15, x_16, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -return x_17; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("note: this linter can be disabled with `set_option ", 51, 51); +return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls_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, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +static lean_object* _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__2() { _start: { -lean_object* x_13; uint8_t x_14; -x_13 = lean_array_get_size(x_2); -x_14 = lean_nat_dec_lt(x_4, x_13); -lean_dec(x_13); -if (x_14 == 0) -{ -lean_object* x_15; -lean_dec(x_4); -lean_dec(x_2); -x_15 = lean_apply_9(x_1, x_3, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -return x_15; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_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; lean_object* x_22; -x_16 = lean_array_fget(x_2, x_4); -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); -x_21 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls_loop___rarg___lambda__1___boxed), 13, 5); -lean_closure_set(x_21, 0, x_4); -lean_closure_set(x_21, 1, x_5); -lean_closure_set(x_21, 2, x_1); -lean_closure_set(x_21, 3, x_2); -lean_closure_set(x_21, 4, x_3); -x_22 = l_Lean_Elab_Term_withAuxDecl___rarg(x_19, x_20, x_18, x_21, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -return x_22; } +static lean_object* _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" false`", 7, 7); +return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls_loop(lean_object* x_1) { +static lean_object* _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__4() { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls_loop___rarg), 12, 0); +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls_loop___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +static lean_object* _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__5() { _start: { -lean_object* x_14; -x_14 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls_loop___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_1); -return x_14; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("\n", 1, 1); +return x_1; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls___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) { +static lean_object* _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__5; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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, 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); +x_11 = !lean_is_exclusive(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); -lean_dec(x_5); -lean_dec(x_4); -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; +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; 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; +x_12 = lean_ctor_get(x_1, 0); +x_13 = lean_ctor_get(x_1, 1); +lean_dec(x_13); +lean_inc(x_12); +x_14 = l_Lean_MessageData_ofName(x_12); +x_15 = l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__2; +lean_ctor_set_tag(x_1, 7); +lean_ctor_set(x_1, 1, x_14); +lean_ctor_set(x_1, 0, x_15); +x_16 = l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__4; +x_17 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_17, 0, x_1); +lean_ctor_set(x_17, 1, x_16); +x_18 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +x_19 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set(x_19, 1, x_3); +x_20 = l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__6; +x_21 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_21, 0, x_19); +lean_ctor_set(x_21, 1, x_20); +x_22 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_22, 0, x_21); +lean_ctor_set(x_22, 1, x_17); +x_23 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_18); +x_24 = lean_alloc_ctor(8, 2, 0); +lean_ctor_set(x_24, 0, x_12); +lean_ctor_set(x_24, 1, x_23); +x_25 = 1; +x_26 = l_Lean_logAt___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__2(x_2, x_24, x_25, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_26; } 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_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_13); -x_16 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkTypeFor(x_13, x_4, x_5, 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; lean_object* x_21; lean_object* x_22; lean_object* x_23; size_t x_24; size_t x_25; lean_object* x_26; -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_13, 0); -lean_inc(x_19); -lean_dec(x_13); -x_20 = lean_ctor_get(x_19, 4); -lean_inc(x_20); -x_21 = lean_ctor_get(x_19, 3); -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_17); -x_23 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_23, 0, x_20); -lean_ctor_set(x_23, 1, x_22); -x_24 = 1; -x_25 = lean_usize_add(x_2, x_24); -x_26 = lean_array_uset(x_15, x_2, x_23); -x_2 = x_25; -x_3 = x_26; -x_10 = x_18; -goto _start; +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; lean_object* x_41; +x_27 = lean_ctor_get(x_1, 0); +lean_inc(x_27); +lean_dec(x_1); +lean_inc(x_27); +x_28 = l_Lean_MessageData_ofName(x_27); +x_29 = l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__2; +x_30 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_30, 0, x_29); +lean_ctor_set(x_30, 1, x_28); +x_31 = l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__4; +x_32 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_31); +x_33 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +x_34 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_34, 0, x_33); +lean_ctor_set(x_34, 1, x_3); +x_35 = l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__6; +x_36 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_36, 0, x_34); +lean_ctor_set(x_36, 1, x_35); +x_37 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_37, 0, x_36); +lean_ctor_set(x_37, 1, x_32); +x_38 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_38, 0, x_37); +lean_ctor_set(x_38, 1, x_33); +x_39 = lean_alloc_ctor(8, 2, 0); +lean_ctor_set(x_39, 0, x_27); +lean_ctor_set(x_39, 1, x_38); +x_40 = 1; +x_41 = l_Lean_logAt___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__2(x_2, x_39, x_40, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_41; } -else +} +} +LEAN_EXPORT lean_object* l_Lean_Linter_logLintIf___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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, lean_object* x_10) { +_start: { -uint8_t x_28; -lean_dec(x_15); -lean_dec(x_13); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -x_28 = !lean_is_exclusive(x_16); -if (x_28 == 0) +lean_object* x_11; uint8_t x_12; +x_11 = lean_ctor_get(x_8, 2); +lean_inc(x_11); +lean_inc(x_1); +x_12 = l_Lean_Linter_getLinterValue(x_1, x_11); +lean_dec(x_11); +if (x_12 == 0) { -return x_16; +lean_object* x_13; lean_object* x_14; +lean_dec(x_8); +lean_dec(x_3); +lean_dec(x_1); +x_13 = lean_box(0); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_13); +lean_ctor_set(x_14, 1, x_10); +return x_14; } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_16, 0); -x_30 = lean_ctor_get(x_16, 1); -lean_inc(x_30); -lean_inc(x_29); -lean_dec(x_16); -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_15; +x_15 = l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_15; } } } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19) { +_start: +{ +lean_object* x_20; lean_object* x_21; +x_20 = lean_alloc_ctor(0, 11, 0); +lean_ctor_set(x_20, 0, x_1); +lean_ctor_set(x_20, 1, x_2); +lean_ctor_set(x_20, 2, x_3); +lean_ctor_set(x_20, 3, x_4); +lean_ctor_set(x_20, 4, x_5); +lean_ctor_set(x_20, 5, x_6); +lean_ctor_set(x_20, 6, x_7); +lean_ctor_set(x_20, 7, x_8); +lean_ctor_set(x_20, 8, x_9); +lean_ctor_set(x_20, 9, x_10); +lean_ctor_set(x_20, 10, x_11); +x_21 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_21, 0, x_20); +lean_ctor_set(x_21, 1, x_19); +return x_21; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls___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) { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1() { _start: { -uint8_t x_13; -x_13 = !lean_is_exclusive(x_10); -if (x_13 == 0) +lean_object* x_1; +x_1 = lean_mk_string_unchecked(":=", 2, 2); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___closed__2() { +_start: { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_14 = lean_ctor_get(x_10, 5); -x_15 = l_Lean_replaceRef(x_1, x_14); -lean_dec(x_14); -lean_ctor_set(x_10, 5, x_15); -x_16 = lean_unsigned_to_nat(0u); -x_17 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls_loop___rarg(x_2, x_3, x_4, x_16, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -return x_17; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("'inductive ... :=' has been deprecated in favor of 'inductive ... where'.", 73, 73); +return x_1; } -else +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___closed__3() { +_start: { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; lean_object* x_30; uint8_t x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_18 = lean_ctor_get(x_10, 0); -x_19 = lean_ctor_get(x_10, 1); -x_20 = lean_ctor_get(x_10, 2); -x_21 = lean_ctor_get(x_10, 3); -x_22 = lean_ctor_get(x_10, 4); -x_23 = lean_ctor_get(x_10, 5); -x_24 = lean_ctor_get(x_10, 6); -x_25 = lean_ctor_get(x_10, 7); -x_26 = lean_ctor_get(x_10, 8); -x_27 = lean_ctor_get(x_10, 9); -x_28 = lean_ctor_get(x_10, 10); -x_29 = lean_ctor_get_uint8(x_10, sizeof(void*)*12); -x_30 = lean_ctor_get(x_10, 11); -x_31 = lean_ctor_get_uint8(x_10, sizeof(void*)*12 + 1); -lean_inc(x_30); -lean_inc(x_28); -lean_inc(x_27); -lean_inc(x_26); -lean_inc(x_25); -lean_inc(x_24); -lean_inc(x_23); -lean_inc(x_22); -lean_inc(x_21); -lean_inc(x_20); -lean_inc(x_19); -lean_inc(x_18); -lean_dec(x_10); -x_32 = l_Lean_replaceRef(x_1, x_23); -lean_dec(x_23); -x_33 = lean_alloc_ctor(0, 12, 2); -lean_ctor_set(x_33, 0, x_18); -lean_ctor_set(x_33, 1, x_19); -lean_ctor_set(x_33, 2, x_20); -lean_ctor_set(x_33, 3, x_21); -lean_ctor_set(x_33, 4, x_22); -lean_ctor_set(x_33, 5, x_32); -lean_ctor_set(x_33, 6, x_24); -lean_ctor_set(x_33, 7, x_25); -lean_ctor_set(x_33, 8, x_26); -lean_ctor_set(x_33, 9, x_27); -lean_ctor_set(x_33, 10, x_28); -lean_ctor_set(x_33, 11, x_30); -lean_ctor_set_uint8(x_33, sizeof(void*)*12, x_29); -lean_ctor_set_uint8(x_33, sizeof(void*)*12 + 1, x_31); -x_34 = lean_unsigned_to_nat(0u); -x_35 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls_loop___rarg(x_2, x_3, x_4, x_34, x_5, x_6, x_7, x_8, x_9, x_33, x_11, x_12); -return x_35; +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___closed__2; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} } +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___closed__3; +x_2 = l_Lean_MessageData_ofFormat(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls___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) { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___closed__5() { _start: { -size_t x_10; size_t x_11; lean_object* x_12; -x_10 = lean_array_size(x_1); -x_11 = 0; -lean_inc(x_8); +lean_object* x_1; +x_1 = l_Lean_Linter_linter_deprecated; +return x_1; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +lean_inc(x_3); +x_10 = l_Lean_Elab_Command_checkValidInductiveModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_10) == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; 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; uint8_t 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; +x_11 = lean_ctor_get(x_10, 1); +lean_inc(x_11); +lean_dec(x_10); +x_12 = lean_unsigned_to_nat(2u); +x_13 = l_Lean_Syntax_getArg(x_2, x_12); +x_14 = l_Lean_Elab_expandOptDeclSig(x_13); +lean_dec(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_unsigned_to_nat(1u); +x_18 = l_Lean_Syntax_getArg(x_2, x_17); +x_19 = lean_ctor_get(x_7, 0); +lean_inc(x_19); +x_20 = lean_ctor_get(x_7, 1); +lean_inc(x_20); +x_21 = lean_ctor_get(x_7, 2); +lean_inc(x_21); +x_22 = lean_ctor_get(x_7, 3); +lean_inc(x_22); +x_23 = lean_ctor_get(x_7, 4); +lean_inc(x_23); +x_24 = lean_ctor_get(x_7, 5); +lean_inc(x_24); +x_25 = lean_ctor_get(x_7, 6); +lean_inc(x_25); +x_26 = lean_ctor_get(x_7, 7); +lean_inc(x_26); +x_27 = lean_ctor_get(x_7, 8); +lean_inc(x_27); +x_28 = lean_ctor_get(x_7, 9); +lean_inc(x_28); +x_29 = lean_ctor_get(x_7, 10); +lean_inc(x_29); +x_30 = lean_ctor_get_uint8(x_7, sizeof(void*)*12); +x_31 = lean_ctor_get(x_7, 11); +lean_inc(x_31); +x_32 = lean_ctor_get_uint8(x_7, sizeof(void*)*12 + 1); +x_33 = l_Lean_Elab_Term_getLevelNames___rarg(x_4, x_5, x_6, x_7, x_8, x_11); +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_7); +lean_inc(x_3); +lean_inc(x_1); +lean_inc(x_25); +x_36 = l_Lean_Elab_Term_expandDeclId(x_25, x_34, x_18, x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_35); +if (lean_obj_tag(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; lean_object* x_46; lean_object* x_47; size_t x_48; size_t x_49; lean_object* x_50; +x_37 = lean_ctor_get(x_36, 0); +lean_inc(x_37); +x_38 = lean_ctor_get(x_36, 1); +lean_inc(x_38); +lean_dec(x_36); +x_39 = lean_ctor_get(x_37, 0); +lean_inc(x_39); +x_40 = lean_ctor_get(x_37, 1); +lean_inc(x_40); +x_41 = lean_ctor_get(x_37, 2); +lean_inc(x_41); +lean_dec(x_37); +x_42 = lean_ctor_get(x_1, 0); +lean_inc(x_42); lean_inc(x_7); +lean_inc(x_2); +lean_inc(x_40); +x_43 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2(x_40, x_42, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_38); +x_44 = lean_ctor_get(x_43, 1); +lean_inc(x_44); +lean_dec(x_43); +x_45 = lean_unsigned_to_nat(4u); +x_46 = l_Lean_Syntax_getArg(x_2, x_45); +x_47 = l_Lean_Syntax_getArgs(x_46); +lean_dec(x_46); +x_48 = lean_array_size(x_47); +x_49 = 0; +lean_inc(x_8); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); +lean_inc(x_40); lean_inc(x_1); -x_12 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls___spec__1(x_10, x_11, x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_12) == 0) +x_50 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23(x_1, x_40, x_48, x_49, x_47, x_3, x_4, x_5, x_6, x_7, x_8, x_44); +if (lean_obj_tag(x_50) == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; -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_1); -x_16 = lean_unsigned_to_nat(0u); -x_17 = lean_nat_dec_lt(x_16, x_15); -lean_dec(x_15); -if (x_17 == 0) +lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; +x_51 = lean_ctor_get(x_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_unsigned_to_nat(5u); +x_54 = l_Lean_Syntax_getArg(x_2, x_53); +x_55 = l_Lean_Syntax_getOptional_x3f(x_54); +lean_dec(x_54); +if (lean_obj_tag(x_55) == 0) { -lean_object* x_28; lean_object* x_29; -lean_dec(x_1); -x_28 = l_Lean_Elab_Command_instInhabitedElabHeaderResult; -x_29 = l_outOfBounds___rarg(x_28); -x_18 = x_29; -goto block_27; +lean_object* x_88; +x_88 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__8___closed__1; +x_56 = x_88; +goto block_87; } else { -lean_object* x_30; -x_30 = lean_array_fget(x_1, x_16); -lean_dec(x_1); -x_18 = x_30; -goto block_27; +lean_object* x_89; lean_object* x_90; lean_object* x_91; +x_89 = lean_ctor_get(x_55, 0); +lean_inc(x_89); +lean_dec(x_55); +x_90 = l_Lean_Syntax_getArg(x_89, x_17); +lean_dec(x_89); +x_91 = l_Lean_Syntax_getArgs(x_90); +lean_dec(x_90); +x_56 = x_91; +goto block_87; } -block_27: +block_87: { -lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_19 = lean_ctor_get(x_18, 3); -lean_inc(x_19); -x_20 = lean_ctor_get(x_18, 1); -lean_inc(x_20); -x_21 = lean_ctor_get(x_18, 2); -lean_inc(x_21); -x_22 = lean_ctor_get(x_18, 0); -lean_inc(x_22); -lean_dec(x_18); -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -lean_dec(x_22); -x_24 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__3___closed__1; -x_25 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls___rarg___lambda__1___boxed), 12, 5); -lean_closure_set(x_25, 0, x_23); -lean_closure_set(x_25, 1, x_2); -lean_closure_set(x_25, 2, x_13); -lean_closure_set(x_25, 3, x_19); -lean_closure_set(x_25, 4, x_24); -x_26 = l_Lean_Meta_withLCtx___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__3___rarg(x_20, x_21, x_25, x_3, x_4, x_5, x_6, x_7, x_8, x_14); -return x_26; -} -} -else +size_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; +x_57 = lean_array_size(x_56); +x_58 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__24(x_57, x_49, x_56, x_3, x_4, x_5, x_6, x_7, x_8, x_52); +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_unsigned_to_nat(6u); +x_62 = l_Lean_Syntax_getArg(x_2, x_61); +lean_inc(x_8); +lean_inc(x_7); +x_63 = l_Lean_Elab_getOptDerivingClasses(x_62, x_7, x_8, x_60); +if (lean_obj_tag(x_63) == 0) { -uint8_t x_31; +lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; uint8_t x_71; +x_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_unsigned_to_nat(3u); +x_67 = l_Lean_Syntax_getArg(x_2, x_66); +x_68 = lean_unsigned_to_nat(0u); +x_69 = l_Lean_Syntax_getArg(x_67, x_68); +x_70 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1; +x_71 = l_Lean_Syntax_isToken(x_70, x_69); +lean_dec(x_69); +if (x_71 == 0) +{ +lean_object* x_72; lean_object* x_73; +lean_dec(x_67); +lean_dec(x_31); +lean_dec(x_29); +lean_dec(x_28); +lean_dec(x_27); +lean_dec(x_26); +lean_dec(x_25); +lean_dec(x_24); +lean_dec(x_23); +lean_dec(x_22); +lean_dec(x_21); +lean_dec(x_20); +lean_dec(x_19); +x_72 = lean_box(0); +x_73 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___lambda__1(x_2, x_18, x_1, x_39, x_40, x_41, x_15, x_16, x_51, x_64, x_59, x_72, x_3, x_4, x_5, x_6, x_7, x_8, x_65); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_31 = !lean_is_exclusive(x_12); -if (x_31 == 0) -{ -return x_12; +return x_73; } else { -lean_object* x_32; lean_object* x_33; lean_object* x_34; -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_alloc_ctor(1, 2, 0); -lean_ctor_set(x_34, 0, x_32); -lean_ctor_set(x_34, 1, x_33); -return x_34; -} -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls___rarg), 9, 0); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls___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_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls___spec__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_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -lean_object* x_13; -x_13 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_1); -return x_13; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isInductiveFamily___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; uint8_t x_12; lean_object* x_13; lean_object* x_14; -x_11 = lean_array_get_size(x_2); -x_12 = lean_nat_dec_lt(x_1, x_11); -lean_dec(x_11); -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_10); -return x_14; -} +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_74 = l_Lean_Syntax_getArg(x_2, x_68); +x_75 = l_Lean_replaceRef(x_74, x_24); +lean_dec(x_24); +lean_dec(x_74); +x_76 = lean_alloc_ctor(0, 12, 2); +lean_ctor_set(x_76, 0, x_19); +lean_ctor_set(x_76, 1, x_20); +lean_ctor_set(x_76, 2, x_21); +lean_ctor_set(x_76, 3, x_22); +lean_ctor_set(x_76, 4, x_23); +lean_ctor_set(x_76, 5, x_75); +lean_ctor_set(x_76, 6, x_25); +lean_ctor_set(x_76, 7, x_26); +lean_ctor_set(x_76, 8, x_27); +lean_ctor_set(x_76, 9, x_28); +lean_ctor_set(x_76, 10, x_29); +lean_ctor_set(x_76, 11, x_31); +lean_ctor_set_uint8(x_76, sizeof(void*)*12, x_30); +lean_ctor_set_uint8(x_76, sizeof(void*)*12 + 1, x_32); +x_77 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___closed__5; +x_78 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___closed__4; +x_79 = l_Lean_Linter_logLintIf___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__25(x_77, x_67, x_78, x_3, x_4, x_5, x_6, x_76, x_8, x_65); +lean_dec(x_67); +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_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___lambda__1(x_2, x_18, x_1, x_39, x_40, x_41, x_15, x_16, x_51, x_64, x_59, x_80, x_3, x_4, x_5, x_6, x_7, x_8, x_81); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_80); +return x_82; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isInductiveFamily(lean_object* x_1, lean_object* x_2, lean_object* x_3, 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); -x_10 = lean_infer_type(x_2, 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; uint8_t x_14; lean_object* x_15; -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_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isInductiveFamily___lambda__1___boxed), 10, 1); -lean_closure_set(x_13, 0, x_1); -x_14 = 0; -x_15 = l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___spec__1___rarg(x_11, x_13, x_14, x_3, x_4, x_5, x_6, x_7, x_8, x_12); -return x_15; } else { -uint8_t x_16; +uint8_t x_83; +lean_dec(x_59); +lean_dec(x_51); +lean_dec(x_41); +lean_dec(x_40); +lean_dec(x_39); +lean_dec(x_31); +lean_dec(x_29); +lean_dec(x_28); +lean_dec(x_27); +lean_dec(x_26); +lean_dec(x_25); +lean_dec(x_24); +lean_dec(x_23); +lean_dec(x_22); +lean_dec(x_21); +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_16); +lean_dec(x_15); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); +lean_dec(x_2); lean_dec(x_1); -x_16 = !lean_is_exclusive(x_10); -if (x_16 == 0) +x_83 = !lean_is_exclusive(x_63); +if (x_83 == 0) { -return x_10; +return x_63; } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; -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_10); -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_84; lean_object* x_85; lean_object* x_86; +x_84 = lean_ctor_get(x_63, 0); +x_85 = lean_ctor_get(x_63, 1); +lean_inc(x_85); +lean_inc(x_84); +lean_dec(x_63); +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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isInductiveFamily___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: +else { -lean_object* x_11; -x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isInductiveFamily___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); +uint8_t x_92; +lean_dec(x_41); +lean_dec(x_40); +lean_dec(x_39); +lean_dec(x_31); +lean_dec(x_29); +lean_dec(x_28); +lean_dec(x_27); +lean_dec(x_26); +lean_dec(x_25); +lean_dec(x_24); +lean_dec(x_23); +lean_dec(x_22); +lean_dec(x_21); +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_16); +lean_dec(x_15); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -5457,1218 +6924,1264 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -return x_11; -} +x_92 = !lean_is_exclusive(x_50); +if (x_92 == 0) +{ +return x_50; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getArrowBinderNames_go(lean_object* x_1, lean_object* x_2) { -_start: +else { -switch (lean_obj_tag(x_1)) { -case 7: +lean_object* x_93; lean_object* x_94; lean_object* x_95; +x_93 = lean_ctor_get(x_50, 0); +x_94 = lean_ctor_get(x_50, 1); +lean_inc(x_94); +lean_inc(x_93); +lean_dec(x_50); +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_3; lean_object* x_4; lean_object* x_5; -x_3 = lean_ctor_get(x_1, 0); -lean_inc(x_3); -x_4 = lean_ctor_get(x_1, 2); -lean_inc(x_4); +uint8_t x_96; +lean_dec(x_31); +lean_dec(x_29); +lean_dec(x_28); +lean_dec(x_27); +lean_dec(x_26); +lean_dec(x_25); +lean_dec(x_24); +lean_dec(x_23); +lean_dec(x_22); +lean_dec(x_21); +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); lean_dec(x_1); -x_5 = lean_array_push(x_2, x_3); -x_1 = x_4; -x_2 = x_5; -goto _start; +x_96 = !lean_is_exclusive(x_36); +if (x_96 == 0) +{ +return x_36; } -case 10: +else { -lean_object* x_7; -x_7 = lean_ctor_get(x_1, 1); -lean_inc(x_7); -lean_dec(x_1); -x_1 = x_7; -goto _start; +lean_object* x_97; lean_object* x_98; lean_object* x_99; +x_97 = lean_ctor_get(x_36, 0); +x_98 = lean_ctor_get(x_36, 1); +lean_inc(x_98); +lean_inc(x_97); +lean_dec(x_36); +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; } -default: +} +} +else { +uint8_t x_100; +lean_dec(x_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; +x_100 = !lean_is_exclusive(x_10); +if (x_100 == 0) +{ +return x_10; +} +else +{ +lean_object* x_101; lean_object* x_102; lean_object* x_103; +x_101 = lean_ctor_get(x_10, 0); +x_102 = lean_ctor_get(x_10, 1); +lean_inc(x_102); +lean_inc(x_101); +lean_dec(x_10); +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_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getArrowBinderNames(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidInductiveModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_2; lean_object* x_3; -x_2 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__3___closed__1; -x_3 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getArrowBinderNames_go(x_1, x_2); -return x_3; +lean_object* x_10; +x_10 = l_Lean_Elab_Command_checkValidInductiveModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +return x_10; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceArrowBinderNames_go(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidInductiveModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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_4; uint8_t x_5; -x_4 = lean_array_get_size(x_1); -x_5 = lean_nat_dec_lt(x_3, x_4); +lean_object* x_9; +x_9 = l_Lean_Elab_Command_checkValidInductiveModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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); -if (x_5 == 0) -{ -return x_2; +lean_dec(x_3); +lean_dec(x_1); +return x_9; } -else -{ -if (lean_obj_tag(x_2) == 7) +} +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: { -lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; uint8_t x_10; -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_ctor_get_uint8(x_2, sizeof(void*)*3 + 8); +lean_object* x_9; +x_9 = l_Lean_Elab_getDeclarationRange_x3f___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); -x_10 = l_Lean_Name_hasMacroScopes(x_6); -if (x_10 == 0) +lean_dec(x_1); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_11 = lean_unsigned_to_nat(1u); -x_12 = lean_nat_add(x_3, x_11); -x_13 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceArrowBinderNames_go(x_1, x_8, x_12); -lean_dec(x_12); -x_14 = l_Lean_Expr_forallE___override(x_6, x_7, x_13, x_9); -return x_14; +lean_object* x_10; +x_10 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_10; } -else +} +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: { -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +lean_object* x_11; +x_11 = l_Lean_Elab_addDeclarationRangesFromSyntax___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_7); lean_dec(x_6); -x_15 = lean_array_fget(x_1, x_3); -x_16 = lean_unsigned_to_nat(1u); -x_17 = lean_nat_add(x_3, x_16); -x_18 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceArrowBinderNames_go(x_1, x_8, x_17); -lean_dec(x_17); -x_19 = l_Lean_Expr_forallE___override(x_15, x_7, x_18, x_9); -return x_19; +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_11; } } -else +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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: { -return x_2; +lean_object* x_12; +x_12 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_12; } } +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_11; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceArrowBinderNames_go___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__12___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_4; -x_4 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceArrowBinderNames_go(x_1, x_2, x_3); +lean_object* x_9; +x_9 = l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__12(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); -return x_4; +return x_9; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceArrowBinderNames(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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) { _start: { -lean_object* x_3; lean_object* x_4; -x_3 = lean_unsigned_to_nat(0u); -x_4 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceArrowBinderNames_go(x_2, x_1, x_3); -return x_4; +lean_object* x_10; +x_10 = l_Lean_throwErrorAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__11(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_1); +return x_10; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceArrowBinderNames___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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) { _start: { -lean_object* x_3; -x_3 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceArrowBinderNames(x_1, x_2); +lean_object* x_9; +x_9 = l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13(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_3; +return x_9; } } -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__1(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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) { _start: { -uint8_t x_5; -x_5 = lean_usize_dec_eq(x_3, x_4); -if (x_5 == 0) -{ -lean_object* x_6; lean_object* x_7; uint8_t x_8; -x_6 = lean_array_uget(x_2, x_3); -x_7 = l_Lean_Expr_fvarId_x21(x_6); +lean_object* x_7; +x_7 = l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__14(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_6); -x_8 = lean_name_eq(x_7, x_1); -lean_dec(x_7); -if (x_8 == 0) +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_liftMacroM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__10___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: { -size_t x_9; size_t x_10; -x_9 = 1; -x_10 = lean_usize_add(x_3, x_9); -x_3 = x_10; -goto _start; +lean_object* x_5; +x_5 = l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__10___lambda__1(x_1, x_2, x_3, x_4); +lean_dec(x_3); +lean_dec(x_1); +return x_5; } -else +} +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__10___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: { -uint8_t x_12; -x_12 = 1; -return x_12; +lean_object* x_5; +x_5 = l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__10___lambda__2(x_1, x_2, x_3, x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_5; } } -else +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__10___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: { -uint8_t x_13; -x_13 = 0; -return x_13; +lean_object* x_7; +x_7 = l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__10___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6); +lean_dec(x_5); +lean_dec(x_1); +return x_7; +} } +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__10___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; +x_7 = l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__10___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6); +lean_dec(x_5); +return x_7; } } -static lean_object* _init_l_Lean_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__2___closed__1() { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(10u); -x_2 = lean_unsigned_to_nat(1u); -x_3 = l_Nat_nextPowerOfTwo_go(x_1, x_2, lean_box(0)); -return x_3; +lean_object* x_9; +x_9 = l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__10(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_9; } } -static lean_object* _init_l_Lean_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__2___closed__2() { +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__15___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__2___closed__1; -x_3 = lean_mk_array(x_2, x_1); -return x_3; +lean_object* x_9; +x_9 = l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__15(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_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__2___closed__3() { +LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__1___boxed(lean_object* x_1) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(0u); -x_2 = l_Lean_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___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); +uint8_t x_2; lean_object* x_3; +x_2 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__1(x_1); +lean_dec(x_1); +x_3 = lean_box(x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___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_EXPORT lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___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: { -if (lean_obj_tag(x_1) == 0) -{ -lean_object* x_9; lean_object* x_10; uint8_t x_11; -x_9 = lean_ctor_get(x_1, 3); -lean_inc(x_9); +uint8_t x_11; lean_object* x_12; +x_11 = lean_unbox(x_1); lean_dec(x_1); -x_10 = lean_st_ref_get(x_5, 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; uint8_t x_16; -x_12 = lean_ctor_get(x_10, 0); -x_13 = lean_ctor_get(x_10, 1); -x_14 = lean_ctor_get(x_12, 0); -lean_inc(x_14); -lean_dec(x_12); -x_15 = l_Lean_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__2___closed__3; -lean_inc(x_14); -lean_ctor_set(x_10, 1, x_14); -lean_ctor_set(x_10, 0, x_15); -x_16 = l_Lean_Expr_hasFVar(x_9); -if (x_16 == 0) -{ -uint8_t x_17; -x_17 = l_Lean_Expr_hasMVar(x_9); -if (x_17 == 0) -{ -lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; -lean_dec(x_10); +x_12 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___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_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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) { +_start: +{ +lean_object* x_9; +x_9 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); +lean_dec(x_1); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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) { +_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_18 = lean_st_ref_take(x_5, 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 = !lean_is_exclusive(x_19); -if (x_21 == 0) +x_13 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_14 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__16(x_1, x_12, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_1); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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_22; lean_object* x_23; uint8_t x_24; -x_22 = lean_ctor_get(x_19, 0); -lean_dec(x_22); -lean_ctor_set(x_19, 0, x_14); -x_23 = lean_st_ref_set(x_5, x_19, x_20); -x_24 = !lean_is_exclusive(x_23); -if (x_24 == 0) +lean_object* x_9; +x_9 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_elabDeclAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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_25; uint8_t x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_23, 0); -lean_dec(x_25); -x_26 = 0; -x_27 = lean_box(x_26); -lean_ctor_set(x_23, 0, x_27); -return x_23; +lean_object* x_9; +x_9 = l_Lean_Elab_elabDeclAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +return x_9; } -else +} +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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) { +_start: { -lean_object* x_28; uint8_t x_29; lean_object* x_30; lean_object* x_31; -x_28 = lean_ctor_get(x_23, 1); -lean_inc(x_28); -lean_dec(x_23); -x_29 = 0; -x_30 = lean_box(x_29); -x_31 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_31, 0, x_30); -lean_ctor_set(x_31, 1, x_28); -return x_31; +lean_object* x_9; +x_9 = l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__18(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; } } -else +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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) { +_start: { -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; lean_object* x_41; lean_object* x_42; -x_32 = lean_ctor_get(x_19, 1); -x_33 = lean_ctor_get(x_19, 2); -x_34 = lean_ctor_get(x_19, 3); -x_35 = lean_ctor_get(x_19, 4); -lean_inc(x_35); -lean_inc(x_34); -lean_inc(x_33); -lean_inc(x_32); -lean_dec(x_19); -x_36 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_36, 0, x_14); -lean_ctor_set(x_36, 1, x_32); -lean_ctor_set(x_36, 2, x_33); -lean_ctor_set(x_36, 3, x_34); -lean_ctor_set(x_36, 4, x_35); -x_37 = lean_st_ref_set(x_5, x_36, x_20); -x_38 = lean_ctor_get(x_37, 1); -lean_inc(x_38); -if (lean_is_exclusive(x_37)) { - lean_ctor_release(x_37, 0); - lean_ctor_release(x_37, 1); - x_39 = x_37; -} else { - lean_dec_ref(x_37); - x_39 = lean_box(0); +lean_object* x_10; +x_10 = l_Lean_throwErrorAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__17(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_1); +return x_10; } -x_40 = 0; -x_41 = lean_box(x_40); -if (lean_is_scalar(x_39)) { - x_42 = lean_alloc_ctor(0, 2, 0); -} else { - x_42 = x_39; } -lean_ctor_set(x_42, 0, x_41); -lean_ctor_set(x_42, 1, x_38); -return x_42; +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__21___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +x_9 = l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__21(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; } } -else +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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) { +_start: { -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_dec(x_14); -x_43 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit(x_2, x_3, x_9, x_10); -x_44 = lean_ctor_get(x_43, 1); -lean_inc(x_44); -x_45 = lean_ctor_get(x_43, 0); -lean_inc(x_45); -lean_dec(x_43); -x_46 = lean_ctor_get(x_44, 1); -lean_inc(x_46); -lean_dec(x_44); -x_47 = lean_st_ref_take(x_5, x_13); -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_is_exclusive(x_48); -if (x_50 == 0) -{ -lean_object* x_51; lean_object* x_52; uint8_t x_53; -x_51 = lean_ctor_get(x_48, 0); -lean_dec(x_51); -lean_ctor_set(x_48, 0, x_46); -x_52 = lean_st_ref_set(x_5, x_48, x_49); -x_53 = !lean_is_exclusive(x_52); -if (x_53 == 0) -{ -lean_object* x_54; -x_54 = lean_ctor_get(x_52, 0); -lean_dec(x_54); -lean_ctor_set(x_52, 0, x_45); -return x_52; +lean_object* x_10; +x_10 = l_Lean_throwErrorAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__20(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_1); +return x_10; } -else +} +LEAN_EXPORT lean_object* l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: { -lean_object* x_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_45); -lean_ctor_set(x_56, 1, x_55); -return x_56; +lean_object* x_9; +x_9 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +return x_9; } } -else +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: { -lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; -x_57 = lean_ctor_get(x_48, 1); -x_58 = lean_ctor_get(x_48, 2); -x_59 = lean_ctor_get(x_48, 3); -x_60 = lean_ctor_get(x_48, 4); -lean_inc(x_60); -lean_inc(x_59); -lean_inc(x_58); -lean_inc(x_57); -lean_dec(x_48); -x_61 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_61, 0, x_46); -lean_ctor_set(x_61, 1, x_57); -lean_ctor_set(x_61, 2, x_58); -lean_ctor_set(x_61, 3, x_59); -lean_ctor_set(x_61, 4, x_60); -x_62 = lean_st_ref_set(x_5, x_61, x_49); -x_63 = lean_ctor_get(x_62, 1); -lean_inc(x_63); -if (lean_is_exclusive(x_62)) { - lean_ctor_release(x_62, 0); - lean_ctor_release(x_62, 1); - x_64 = x_62; -} else { - lean_dec_ref(x_62); - x_64 = lean_box(0); -} -if (lean_is_scalar(x_64)) { - x_65 = lean_alloc_ctor(0, 2, 0); -} else { - x_65 = x_64; +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_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__1(x_1, x_2, x_3, x_4, x_15, x_16, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_2); +lean_dec(x_1); +return x_17; } -lean_ctor_set(x_65, 0, x_45); -lean_ctor_set(x_65, 1, x_63); -return x_65; } +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, 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_7); +lean_dec(x_7); +x_17 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__2(x_1, x_2, x_3, x_4, x_15, x_6, x_16, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_13); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_2); +lean_dec(x_1); +return x_17; } } -else -{ -lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; uint8_t x_73; -lean_dec(x_14); -x_66 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit(x_2, x_3, x_9, x_10); -x_67 = lean_ctor_get(x_66, 1); -lean_inc(x_67); -x_68 = lean_ctor_get(x_66, 0); -lean_inc(x_68); -lean_dec(x_66); -x_69 = lean_ctor_get(x_67, 1); -lean_inc(x_69); -lean_dec(x_67); -x_70 = lean_st_ref_take(x_5, x_13); -x_71 = lean_ctor_get(x_70, 0); -lean_inc(x_71); -x_72 = lean_ctor_get(x_70, 1); -lean_inc(x_72); -lean_dec(x_70); -x_73 = !lean_is_exclusive(x_71); -if (x_73 == 0) +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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, lean_object* x_7, lean_object* x_8, 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_74; lean_object* x_75; uint8_t x_76; -x_74 = lean_ctor_get(x_71, 0); -lean_dec(x_74); -lean_ctor_set(x_71, 0, x_69); -x_75 = lean_st_ref_set(x_5, x_71, x_72); -x_76 = !lean_is_exclusive(x_75); -if (x_76 == 0) +uint8_t x_15; lean_object* x_16; +x_15 = lean_unbox(x_4); +lean_dec(x_4); +x_16 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3(x_1, x_2, x_3, x_15, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_13); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +lean_dec(x_1); +return x_16; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: { -lean_object* x_77; -x_77 = lean_ctor_get(x_75, 0); -lean_dec(x_77); -lean_ctor_set(x_75, 0, x_68); -return x_75; +lean_object* x_9; +x_9 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_9; } -else +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__22___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, 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_78; lean_object* x_79; -x_78 = lean_ctor_get(x_75, 1); -lean_inc(x_78); -lean_dec(x_75); -x_79 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_79, 0, x_68); -lean_ctor_set(x_79, 1, x_78); -return x_79; +lean_object* x_10; +x_10 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__22___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +return x_10; } } -else +LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__22___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_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; -x_80 = lean_ctor_get(x_71, 1); -x_81 = lean_ctor_get(x_71, 2); -x_82 = lean_ctor_get(x_71, 3); -x_83 = lean_ctor_get(x_71, 4); -lean_inc(x_83); -lean_inc(x_82); -lean_inc(x_81); -lean_inc(x_80); -lean_dec(x_71); -x_84 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_84, 0, x_69); -lean_ctor_set(x_84, 1, x_80); -lean_ctor_set(x_84, 2, x_81); -lean_ctor_set(x_84, 3, x_82); -lean_ctor_set(x_84, 4, x_83); -x_85 = lean_st_ref_set(x_5, x_84, x_72); -x_86 = lean_ctor_get(x_85, 1); -lean_inc(x_86); -if (lean_is_exclusive(x_85)) { - lean_ctor_release(x_85, 0); - lean_ctor_release(x_85, 1); - x_87 = x_85; -} else { - lean_dec_ref(x_85); - x_87 = lean_box(0); +lean_object* x_10; +x_10 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__22___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +return x_10; } -if (lean_is_scalar(x_87)) { - x_88 = lean_alloc_ctor(0, 2, 0); -} else { - x_88 = x_87; } -lean_ctor_set(x_88, 0, x_68); -lean_ctor_set(x_88, 1, x_86); -return x_88; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__22___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__22___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +return x_10; } } +LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__22___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +x_9 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__22(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); +return x_9; } -else +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: { -lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; uint8_t x_94; -x_89 = lean_ctor_get(x_10, 0); -x_90 = lean_ctor_get(x_10, 1); -lean_inc(x_90); -lean_inc(x_89); +lean_object* x_12; +x_12 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_10); -x_91 = lean_ctor_get(x_89, 0); -lean_inc(x_91); -lean_dec(x_89); -x_92 = l_Lean_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__2___closed__3; -lean_inc(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_91); -x_94 = l_Lean_Expr_hasFVar(x_9); -if (x_94 == 0) +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_4); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___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: { -uint8_t x_95; -x_95 = l_Lean_Expr_hasMVar(x_9); -if (x_95 == 0) +lean_object* x_13; +x_13 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_11); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_4); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: { -lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; uint8_t x_108; lean_object* x_109; lean_object* x_110; -lean_dec(x_93); +lean_object* x_13; +x_13 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_11); lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_5); lean_dec(x_3); -lean_dec(x_2); -x_96 = lean_st_ref_take(x_5, x_90); -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_ctor_get(x_97, 1); -lean_inc(x_99); -x_100 = lean_ctor_get(x_97, 2); -lean_inc(x_100); -x_101 = lean_ctor_get(x_97, 3); -lean_inc(x_101); -x_102 = lean_ctor_get(x_97, 4); -lean_inc(x_102); -if (lean_is_exclusive(x_97)) { - lean_ctor_release(x_97, 0); - lean_ctor_release(x_97, 1); - lean_ctor_release(x_97, 2); - lean_ctor_release(x_97, 3); - lean_ctor_release(x_97, 4); - x_103 = x_97; -} else { - lean_dec_ref(x_97); - x_103 = lean_box(0); -} -if (lean_is_scalar(x_103)) { - x_104 = lean_alloc_ctor(0, 5, 0); -} else { - x_104 = x_103; +return x_13; } -lean_ctor_set(x_104, 0, x_91); -lean_ctor_set(x_104, 1, x_99); -lean_ctor_set(x_104, 2, x_100); -lean_ctor_set(x_104, 3, x_101); -lean_ctor_set(x_104, 4, x_102); -x_105 = lean_st_ref_set(x_5, x_104, x_98); -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 = 0; -x_109 = lean_box(x_108); -if (lean_is_scalar(x_107)) { - x_110 = lean_alloc_ctor(0, 2, 0); -} else { - x_110 = x_107; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +x_12 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_4); +lean_dec(x_1); +return x_12; } -lean_ctor_set(x_110, 0, x_109); -lean_ctor_set(x_110, 1, x_106); -return x_110; } -else +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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: { -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_dec(x_91); -x_111 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit(x_2, x_3, x_9, x_93); -x_112 = lean_ctor_get(x_111, 1); -lean_inc(x_112); -x_113 = lean_ctor_get(x_111, 0); -lean_inc(x_113); -lean_dec(x_111); -x_114 = lean_ctor_get(x_112, 1); -lean_inc(x_114); -lean_dec(x_112); -x_115 = lean_st_ref_take(x_5, x_90); -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, 1); -lean_inc(x_118); -x_119 = lean_ctor_get(x_116, 2); -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); -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); - x_122 = x_116; -} else { - lean_dec_ref(x_116); - x_122 = lean_box(0); +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_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23(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_10); +return x_15; } -if (lean_is_scalar(x_122)) { - x_123 = lean_alloc_ctor(0, 5, 0); -} else { - x_123 = x_122; } -lean_ctor_set(x_123, 0, x_114); -lean_ctor_set(x_123, 1, x_118); -lean_ctor_set(x_123, 2, x_119); -lean_ctor_set(x_123, 3, x_120); -lean_ctor_set(x_123, 4, x_121); -x_124 = lean_st_ref_set(x_5, x_123, x_117); -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_124); - x_126 = lean_box(0); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__24___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, 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_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__24(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_4); +return x_13; } -if (lean_is_scalar(x_126)) { - x_127 = lean_alloc_ctor(0, 2, 0); -} else { - x_127 = x_126; } -lean_ctor_set(x_127, 0, x_113); -lean_ctor_set(x_127, 1, x_125); -return x_127; +LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +return x_11; } } -else +LEAN_EXPORT lean_object* l_Lean_Linter_logLintIf___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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_object* x_10) { +_start: { -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_dec(x_91); -x_128 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit(x_2, x_3, x_9, x_93); -x_129 = lean_ctor_get(x_128, 1); -lean_inc(x_129); -x_130 = lean_ctor_get(x_128, 0); -lean_inc(x_130); -lean_dec(x_128); -x_131 = lean_ctor_get(x_129, 1); -lean_inc(x_131); -lean_dec(x_129); -x_132 = lean_st_ref_take(x_5, x_90); -x_133 = lean_ctor_get(x_132, 0); -lean_inc(x_133); -x_134 = lean_ctor_get(x_132, 1); -lean_inc(x_134); -lean_dec(x_132); -x_135 = lean_ctor_get(x_133, 1); -lean_inc(x_135); -x_136 = lean_ctor_get(x_133, 2); -lean_inc(x_136); -x_137 = lean_ctor_get(x_133, 3); -lean_inc(x_137); -x_138 = lean_ctor_get(x_133, 4); -lean_inc(x_138); -if (lean_is_exclusive(x_133)) { - lean_ctor_release(x_133, 0); - lean_ctor_release(x_133, 1); - lean_ctor_release(x_133, 2); - lean_ctor_release(x_133, 3); - lean_ctor_release(x_133, 4); - x_139 = x_133; -} else { - lean_dec_ref(x_133); - x_139 = lean_box(0); +lean_object* x_11; +x_11 = l_Lean_Linter_logLintIf___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__25(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +return x_11; } -if (lean_is_scalar(x_139)) { - x_140 = lean_alloc_ctor(0, 5, 0); -} else { - x_140 = x_139; -} -lean_ctor_set(x_140, 0, x_131); -lean_ctor_set(x_140, 1, x_135); -lean_ctor_set(x_140, 2, x_136); -lean_ctor_set(x_140, 3, x_137); -lean_ctor_set(x_140, 4, x_138); -x_141 = lean_st_ref_set(x_5, x_140, x_134); -x_142 = lean_ctor_get(x_141, 1); -lean_inc(x_142); -if (lean_is_exclusive(x_141)) { - lean_ctor_release(x_141, 0); - lean_ctor_release(x_141, 1); - x_143 = x_141; -} else { - lean_dec_ref(x_141); - x_143 = lean_box(0); -} -if (lean_is_scalar(x_143)) { - x_144 = lean_alloc_ctor(0, 2, 0); -} else { - x_144 = x_143; -} -lean_ctor_set(x_144, 0, x_130); -lean_ctor_set(x_144, 1, x_142); -return x_144; } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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_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); +return x_20; } } -else -{ -lean_object* x_145; lean_object* x_146; lean_object* x_147; uint8_t x_148; -x_145 = lean_ctor_get(x_1, 3); -lean_inc(x_145); -x_146 = lean_ctor_get(x_1, 4); -lean_inc(x_146); -lean_dec(x_1); -x_147 = lean_st_ref_get(x_5, x_8); -x_148 = !lean_is_exclusive(x_147); -if (x_148 == 0) +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___spec__1(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4) { +_start: { -lean_object* x_149; lean_object* x_150; lean_object* x_151; uint8_t x_152; lean_object* x_153; uint8_t x_178; lean_object* x_179; lean_object* x_192; uint8_t x_193; -x_149 = lean_ctor_get(x_147, 0); -x_150 = lean_ctor_get(x_147, 1); -x_151 = lean_ctor_get(x_149, 0); -lean_inc(x_151); -lean_dec(x_149); -x_192 = l_Lean_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__2___closed__3; -lean_ctor_set(x_147, 1, x_151); -lean_ctor_set(x_147, 0, x_192); -x_193 = l_Lean_Expr_hasFVar(x_145); -if (x_193 == 0) +uint8_t x_5; +x_5 = lean_usize_dec_eq(x_3, x_4); +if (x_5 == 0) { -uint8_t x_194; -x_194 = l_Lean_Expr_hasMVar(x_145); -if (x_194 == 0) +lean_object* x_6; lean_object* x_7; uint8_t x_8; +x_6 = lean_array_uget(x_2, x_3); +x_7 = lean_ctor_get(x_6, 3); +lean_inc(x_7); +lean_dec(x_6); +x_8 = lean_name_eq(x_7, x_1); +lean_dec(x_7); +if (x_8 == 0) { -uint8_t x_195; -lean_dec(x_145); -x_195 = 0; -x_178 = x_195; -x_179 = x_147; -goto block_191; +size_t x_9; size_t x_10; +x_9 = 1; +x_10 = lean_usize_add(x_3, x_9); +x_3 = x_10; +goto _start; } else { -lean_object* x_196; lean_object* x_197; lean_object* x_198; uint8_t x_199; -lean_inc(x_3); -lean_inc(x_2); -x_196 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit(x_2, x_3, x_145, x_147); -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_unbox(x_197); -lean_dec(x_197); -x_178 = x_199; -x_179 = x_198; -goto block_191; +uint8_t x_12; +x_12 = 1; +return x_12; } } else { -lean_object* x_200; lean_object* x_201; lean_object* x_202; uint8_t x_203; -lean_inc(x_3); -lean_inc(x_2); -x_200 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit(x_2, x_3, x_145, x_147); -x_201 = lean_ctor_get(x_200, 0); -lean_inc(x_201); -x_202 = lean_ctor_get(x_200, 1); -lean_inc(x_202); -lean_dec(x_200); -x_203 = lean_unbox(x_201); -lean_dec(x_201); -x_178 = x_203; -x_179 = x_202; -goto block_191; +uint8_t x_13; +x_13 = 0; +return x_13; } -block_177: -{ -lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; uint8_t x_158; -x_154 = lean_ctor_get(x_153, 1); -lean_inc(x_154); -lean_dec(x_153); -x_155 = lean_st_ref_take(x_5, x_150); -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_is_exclusive(x_156); -if (x_158 == 0) +} +} +LEAN_EXPORT uint8_t l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__1(lean_object* x_1, lean_object* x_2) { +_start: { -lean_object* x_159; lean_object* x_160; uint8_t x_161; -x_159 = lean_ctor_get(x_156, 0); -lean_dec(x_159); -lean_ctor_set(x_156, 0, x_154); -x_160 = lean_st_ref_set(x_5, x_156, x_157); -x_161 = !lean_is_exclusive(x_160); -if (x_161 == 0) +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) { -lean_object* x_162; lean_object* x_163; -x_162 = lean_ctor_get(x_160, 0); -lean_dec(x_162); -x_163 = lean_box(x_152); -lean_ctor_set(x_160, 0, x_163); -return x_160; +uint8_t x_6; +lean_dec(x_3); +x_6 = 0; +return x_6; } else { -lean_object* x_164; lean_object* x_165; lean_object* x_166; -x_164 = lean_ctor_get(x_160, 1); -lean_inc(x_164); -lean_dec(x_160); -x_165 = lean_box(x_152); -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; +size_t x_7; size_t x_8; uint8_t x_9; +x_7 = 0; +x_8 = lean_usize_of_nat(x_3); +lean_dec(x_3); +x_9 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___spec__1(x_2, x_1, x_7, x_8); +return x_9; } } -else +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: { -lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; -x_167 = lean_ctor_get(x_156, 1); -x_168 = lean_ctor_get(x_156, 2); -x_169 = lean_ctor_get(x_156, 3); -x_170 = lean_ctor_get(x_156, 4); -lean_inc(x_170); -lean_inc(x_169); -lean_inc(x_168); -lean_inc(x_167); -lean_dec(x_156); -x_171 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_171, 0, x_154); -lean_ctor_set(x_171, 1, x_167); -lean_ctor_set(x_171, 2, x_168); -lean_ctor_set(x_171, 3, x_169); -lean_ctor_set(x_171, 4, x_170); -x_172 = lean_st_ref_set(x_5, x_171, x_157); -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_172); - x_174 = lean_box(0); +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_12 = l_Lean_Elab_Term_getLevelNames___rarg(x_6, x_7, x_8, x_9, x_10, x_11); +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_12, 1); +lean_inc(x_14); +lean_dec(x_12); +x_15 = lean_ctor_get(x_7, 1); +x_16 = l_Lean_Meta_getLocalInstances(x_7, x_8, x_9, x_10, x_14); +x_17 = !lean_is_exclusive(x_16); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_16, 0); +lean_inc(x_15); +x_19 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_19, 0, x_1); +lean_ctor_set(x_19, 1, x_15); +lean_ctor_set(x_19, 2, x_18); +lean_ctor_set(x_19, 3, x_13); +lean_ctor_set(x_19, 4, x_3); +lean_ctor_set(x_19, 5, x_4); +x_20 = lean_array_push(x_2, x_19); +lean_ctor_set(x_16, 0, x_20); +return x_16; } -x_175 = lean_box(x_152); -if (lean_is_scalar(x_174)) { - x_176 = lean_alloc_ctor(0, 2, 0); -} else { - x_176 = x_174; +else +{ +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_16, 0); +x_22 = lean_ctor_get(x_16, 1); +lean_inc(x_22); +lean_inc(x_21); +lean_dec(x_16); +lean_inc(x_15); +x_23 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_23, 0, x_1); +lean_ctor_set(x_23, 1, x_15); +lean_ctor_set(x_23, 2, x_21); +lean_ctor_set(x_23, 3, x_13); +lean_ctor_set(x_23, 4, x_3); +lean_ctor_set(x_23, 5, x_4); +x_24 = lean_array_push(x_2, x_23); +x_25 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_25, 0, x_24); +lean_ctor_set(x_25, 1, x_22); +return x_25; } -lean_ctor_set(x_176, 0, x_175); -lean_ctor_set(x_176, 1, x_173); -return x_176; } } -block_191: +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___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: { -if (x_178 == 0) +uint8_t x_10; uint8_t x_11; lean_object* x_12; +x_10 = 1; +x_11 = 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_12 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_10, x_11, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_12) == 0) { -uint8_t x_180; -x_180 = l_Lean_Expr_hasFVar(x_146); -if (x_180 == 0) +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_12, 1); +lean_inc(x_13); +lean_dec(x_12); +x_14 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__8___closed__1; +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_15 = l_Lean_Elab_Term_addAutoBoundImplicits(x_14, x_3, x_4, x_5, x_6, x_7, x_8, x_13); +lean_dec(x_4); +if (lean_obj_tag(x_15) == 0) { -uint8_t x_181; -x_181 = l_Lean_Expr_hasMVar(x_146); -if (x_181 == 0) +lean_object* x_16; lean_object* x_17; uint8_t x_18; uint8_t x_19; lean_object* 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 = 1; +x_19 = 1; +lean_inc(x_16); +x_20 = l_Lean_Meta_mkForallFVars(x_16, x_1, x_11, x_18, x_19, x_5, x_6, x_7, x_8, x_17); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +if (lean_obj_tag(x_20) == 0) { -uint8_t x_182; -lean_dec(x_146); -lean_dec(x_3); -lean_dec(x_2); -x_182 = 0; -x_152 = x_182; -x_153 = x_179; -goto block_177; +uint8_t x_21; +x_21 = !lean_is_exclusive(x_20); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_20, 0); +x_23 = lean_array_get_size(x_16); +lean_dec(x_16); +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); +lean_ctor_set(x_20, 0, x_24); +return x_20; } else { -lean_object* x_183; lean_object* x_184; lean_object* x_185; uint8_t x_186; -x_183 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit(x_2, x_3, x_146, x_179); -x_184 = lean_ctor_get(x_183, 0); -lean_inc(x_184); -x_185 = lean_ctor_get(x_183, 1); -lean_inc(x_185); -lean_dec(x_183); -x_186 = lean_unbox(x_184); -lean_dec(x_184); -x_152 = x_186; -x_153 = x_185; -goto block_177; +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_20, 0); +x_26 = lean_ctor_get(x_20, 1); +lean_inc(x_26); +lean_inc(x_25); +lean_dec(x_20); +x_27 = lean_array_get_size(x_16); +lean_dec(x_16); +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_29 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_26); +return x_29; } } else { -lean_object* x_187; lean_object* x_188; lean_object* x_189; uint8_t x_190; -x_187 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit(x_2, x_3, x_146, x_179); -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); -x_190 = lean_unbox(x_188); -lean_dec(x_188); -x_152 = x_190; -x_153 = x_189; -goto block_177; -} +uint8_t x_30; +lean_dec(x_16); +x_30 = !lean_is_exclusive(x_20); +if (x_30 == 0) +{ +return x_20; } else { -lean_dec(x_146); -lean_dec(x_3); -lean_dec(x_2); -x_152 = x_178; -x_153 = x_179; -goto block_177; +lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_31 = lean_ctor_get(x_20, 0); +x_32 = lean_ctor_get(x_20, 1); +lean_inc(x_32); +lean_inc(x_31); +lean_dec(x_20); +x_33 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_33, 0, x_31); +lean_ctor_set(x_33, 1, x_32); +return x_33; } } } else { -lean_object* x_204; lean_object* x_205; lean_object* x_206; uint8_t x_207; lean_object* x_208; uint8_t x_225; lean_object* x_226; lean_object* x_239; lean_object* x_240; uint8_t x_241; -x_204 = lean_ctor_get(x_147, 0); -x_205 = lean_ctor_get(x_147, 1); -lean_inc(x_205); -lean_inc(x_204); -lean_dec(x_147); -x_206 = lean_ctor_get(x_204, 0); -lean_inc(x_206); -lean_dec(x_204); -x_239 = l_Lean_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__2___closed__3; -x_240 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_240, 0, x_239); -lean_ctor_set(x_240, 1, x_206); -x_241 = l_Lean_Expr_hasFVar(x_145); -if (x_241 == 0) -{ -uint8_t x_242; -x_242 = l_Lean_Expr_hasMVar(x_145); -if (x_242 == 0) +uint8_t x_34; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_1); +x_34 = !lean_is_exclusive(x_15); +if (x_34 == 0) { -uint8_t x_243; -lean_dec(x_145); -x_243 = 0; -x_225 = x_243; -x_226 = x_240; -goto block_238; +return x_15; } else { -lean_object* x_244; lean_object* x_245; lean_object* x_246; uint8_t x_247; -lean_inc(x_3); -lean_inc(x_2); -x_244 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit(x_2, x_3, x_145, x_240); -x_245 = lean_ctor_get(x_244, 0); -lean_inc(x_245); -x_246 = lean_ctor_get(x_244, 1); -lean_inc(x_246); -lean_dec(x_244); -x_247 = lean_unbox(x_245); -lean_dec(x_245); -x_225 = x_247; -x_226 = x_246; -goto block_238; +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_15, 0); +x_36 = lean_ctor_get(x_15, 1); +lean_inc(x_36); +lean_inc(x_35); +lean_dec(x_15); +x_37 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +return x_37; +} } } else { -lean_object* x_248; lean_object* x_249; lean_object* x_250; uint8_t x_251; -lean_inc(x_3); -lean_inc(x_2); -x_248 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit(x_2, x_3, x_145, x_240); -x_249 = lean_ctor_get(x_248, 0); -lean_inc(x_249); -x_250 = lean_ctor_get(x_248, 1); -lean_inc(x_250); -lean_dec(x_248); -x_251 = lean_unbox(x_249); -lean_dec(x_249); -x_225 = x_251; -x_226 = x_250; -goto block_238; +uint8_t x_38; +lean_dec(x_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_38 = !lean_is_exclusive(x_12); +if (x_38 == 0) +{ +return x_12; } -block_224: +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; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; -x_209 = lean_ctor_get(x_208, 1); -lean_inc(x_209); -lean_dec(x_208); -x_210 = lean_st_ref_take(x_5, x_205); -x_211 = lean_ctor_get(x_210, 0); -lean_inc(x_211); -x_212 = lean_ctor_get(x_210, 1); -lean_inc(x_212); -lean_dec(x_210); -x_213 = lean_ctor_get(x_211, 1); -lean_inc(x_213); -x_214 = lean_ctor_get(x_211, 2); -lean_inc(x_214); -x_215 = lean_ctor_get(x_211, 3); -lean_inc(x_215); -x_216 = lean_ctor_get(x_211, 4); -lean_inc(x_216); -if (lean_is_exclusive(x_211)) { - lean_ctor_release(x_211, 0); - lean_ctor_release(x_211, 1); - lean_ctor_release(x_211, 2); - lean_ctor_release(x_211, 3); - lean_ctor_release(x_211, 4); - x_217 = x_211; -} else { - lean_dec_ref(x_211); - x_217 = lean_box(0); +lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = lean_ctor_get(x_12, 0); +x_40 = lean_ctor_get(x_12, 1); +lean_inc(x_40); +lean_inc(x_39); +lean_dec(x_12); +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; } -if (lean_is_scalar(x_217)) { - x_218 = lean_alloc_ctor(0, 5, 0); -} else { - x_218 = x_217; } -lean_ctor_set(x_218, 0, x_209); -lean_ctor_set(x_218, 1, x_213); -lean_ctor_set(x_218, 2, x_214); -lean_ctor_set(x_218, 3, x_215); -lean_ctor_set(x_218, 4, x_216); -x_219 = lean_st_ref_set(x_5, x_218, x_212); -x_220 = lean_ctor_get(x_219, 1); -lean_inc(x_220); -if (lean_is_exclusive(x_219)) { - lean_ctor_release(x_219, 0); - lean_ctor_release(x_219, 1); - x_221 = x_219; -} else { - lean_dec_ref(x_219); - x_221 = lean_box(0); } -x_222 = lean_box(x_207); -if (lean_is_scalar(x_221)) { - x_223 = lean_alloc_ctor(0, 2, 0); -} else { - x_223 = x_221; } -lean_ctor_set(x_223, 0, x_222); -lean_ctor_set(x_223, 1, x_220); -return x_223; +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__4___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("invalid inductive type, resultant type is not a sort", 52, 52); +return x_1; } -block_238: +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__4___closed__2() { +_start: { -if (x_225 == 0) +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__4___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: { -uint8_t x_227; -x_227 = l_Lean_Expr_hasFVar(x_146); -if (x_227 == 0) +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); +lean_inc(x_1); +x_9 = l_Lean_Elab_Term_elabType(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_9) == 0) { -uint8_t x_228; -x_228 = l_Lean_Expr_hasMVar(x_146); -if (x_228 == 0) +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_9, 0); +lean_inc(x_10); +x_11 = lean_ctor_get(x_9, 1); +lean_inc(x_11); +lean_dec(x_9); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_10); +x_12 = l_Lean_Meta_isTypeFormerType(x_10, x_4, x_5, x_6, x_7, x_11); +if (lean_obj_tag(x_12) == 0) { -uint8_t x_229; -lean_dec(x_146); +lean_object* x_13; uint8_t x_14; +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_unbox(x_13); +lean_dec(x_13); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; +lean_dec(x_10); +x_15 = lean_ctor_get(x_12, 1); +lean_inc(x_15); +lean_dec(x_12); +x_16 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__4___closed__2; +x_17 = l_Lean_throwErrorAt___at___private_Lean_Elab_Binders_0__Lean_Elab_Term_elabBinderViews_loop___spec__1(x_1, x_16, x_2, x_3, x_4, x_5, x_6, x_7, x_15); +lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); -x_229 = 0; -x_207 = x_229; -x_208 = x_226; -goto block_224; +lean_dec(x_1); +x_18 = !lean_is_exclusive(x_17); +if (x_18 == 0) +{ +return x_17; } else { -lean_object* x_230; lean_object* x_231; lean_object* x_232; uint8_t x_233; -x_230 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit(x_2, x_3, x_146, x_226); -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); -x_233 = lean_unbox(x_231); -lean_dec(x_231); -x_207 = x_233; -x_208 = x_232; -goto block_224; +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(1, 2, 0); +lean_ctor_set(x_21, 0, x_19); +lean_ctor_set(x_21, 1, x_20); +return x_21; } } else { -lean_object* x_234; lean_object* x_235; lean_object* x_236; uint8_t x_237; -x_234 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit(x_2, x_3, x_146, x_226); -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_unbox(x_235); -lean_dec(x_235); -x_207 = x_237; -x_208 = x_236; -goto block_224; +lean_object* x_22; lean_object* x_23; lean_object* x_24; +lean_dec(x_1); +x_22 = lean_ctor_get(x_12, 1); +lean_inc(x_22); +lean_dec(x_12); +x_23 = lean_box(0); +x_24 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__3(x_10, x_23, x_2, x_3, x_4, x_5, x_6, x_7, x_22); +return x_24; } } else { -lean_dec(x_146); +uint8_t x_25; +lean_dec(x_10); +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_207 = x_225; -x_208 = x_226; -goto block_224; -} -} +lean_dec(x_1); +x_25 = !lean_is_exclusive(x_12); +if (x_25 == 0) +{ +return x_12; } +else +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_12, 0); +x_27 = lean_ctor_get(x_12, 1); +lean_inc(x_27); +lean_inc(x_26); +lean_dec(x_12); +x_28 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +return x_28; } } } -LEAN_EXPORT lean_object* l_Array_erase___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__3(lean_object* x_1, lean_object* x_2) { -_start: +else { -lean_object* x_3; lean_object* x_4; -x_3 = lean_unsigned_to_nat(0u); -x_4 = l_Array_indexOfAux___at___private_Lean_Meta_Constructions_BRecOn_0__Lean_buildBRecOnMinorPremise_go___spec__1(x_1, x_2, x_3); -if (lean_obj_tag(x_4) == 0) +uint8_t x_29; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_29 = !lean_is_exclusive(x_9); +if (x_29 == 0) { -return x_1; +return x_9; } else { -lean_object* x_5; lean_object* x_6; -x_5 = lean_ctor_get(x_4, 0); -lean_inc(x_5); -lean_dec(x_4); -x_6 = l_Array_feraseIdx___rarg(x_1, x_5); -return x_6; +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_9, 0); +x_31 = lean_ctor_get(x_9, 1); +lean_inc(x_31); +lean_inc(x_30); +lean_dec(x_9); +x_32 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_31); +return x_32; } } } -LEAN_EXPORT uint8_t l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__1(lean_object* x_1, lean_object* x_2) { +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_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) +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_13 = l_Lean_Elab_Term_getLevelNames___rarg(x_7, x_8, x_9, x_10, x_11, x_12); +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_13, 1); +lean_inc(x_15); +lean_dec(x_13); +x_16 = lean_ctor_get(x_8, 1); +x_17 = l_Lean_Meta_getLocalInstances(x_8, x_9, x_10, x_11, x_15); +x_18 = !lean_is_exclusive(x_17); +if (x_18 == 0) { -uint8_t x_6; -lean_dec(x_3); -x_6 = 0; -return x_6; +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_17, 0); +lean_inc(x_16); +x_20 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_20, 0, x_1); +lean_ctor_set(x_20, 1, x_16); +lean_ctor_set(x_20, 2, x_19); +lean_ctor_set(x_20, 3, x_14); +lean_ctor_set(x_20, 4, x_2); +lean_ctor_set(x_20, 5, x_3); +x_21 = lean_array_push(x_4, x_20); +lean_ctor_set(x_17, 0, x_21); +return x_17; } else { -size_t x_7; size_t x_8; uint8_t x_9; -x_7 = 0; -x_8 = lean_usize_of_nat(x_3); -lean_dec(x_3); -x_9 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__1(x_2, x_1, x_7, x_8); -return x_9; +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_22 = lean_ctor_get(x_17, 0); +x_23 = lean_ctor_get(x_17, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_17); +lean_inc(x_16); +x_24 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_24, 0, x_1); +lean_ctor_set(x_24, 1, x_16); +lean_ctor_set(x_24, 2, x_22); +lean_ctor_set(x_24, 3, x_14); +lean_ctor_set(x_24, 4, x_2); +lean_ctor_set(x_24, 5, x_3); +x_25 = lean_array_push(x_4, x_24); +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_23); +return x_26; } } } -LEAN_EXPORT uint8_t l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__2(lean_object* x_1) { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__1() { _start: { -uint8_t x_2; -x_2 = 0; -return x_2; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("header params: ", 15, 15); +return x_1; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___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) { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__2() { _start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -lean_inc(x_1); -x_10 = lean_array_push(x_3, x_1); -x_11 = l_Array_erase___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__3(x_2, x_1); -lean_dec(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_10); -x_13 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_13, 0, x_12); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_13); -lean_ctor_set(x_14, 1, x_9); -return x_14; +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__4___closed__1() { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__3() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__2___boxed), 1, 0); +x_1 = lean_mk_string_unchecked(", type: ", 8, 8); return x_1; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__4() { _start: { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; -lean_inc(x_3); -x_11 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__1___boxed), 2, 1); -lean_closure_set(x_11, 0, x_3); -x_12 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__4___closed__1; -x_13 = l_Lean_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__2(x_1, x_11, x_12, x_6, x_7, x_8, x_9, x_10); +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___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; uint8_t x_15; +x_12 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__3; +x_13 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_12, x_5, x_6, x_7, x_8, x_9, x_10, x_11); x_14 = lean_ctor_get(x_13, 0); lean_inc(x_14); x_15 = lean_unbox(x_14); @@ -6680,3682 +8193,3235 @@ x_16 = lean_ctor_get(x_13, 1); lean_inc(x_16); lean_dec(x_13); x_17 = lean_box(0); -x_18 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__3(x_2, x_3, x_4, x_17, x_6, x_7, x_8, x_9, x_16); +x_18 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__5(x_1, x_3, x_4, x_2, x_17, x_5, x_6, x_7, x_8, x_9, x_10, x_16); return x_18; } else { uint8_t x_19; -lean_dec(x_2); x_19 = !lean_is_exclusive(x_13); if (x_19 == 0) { -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_13, 0); -lean_dec(x_20); -x_21 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_21, 0, x_3); -lean_ctor_set(x_21, 1, x_4); -x_22 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_22, 0, x_21); -lean_ctor_set(x_13, 0, x_22); -return x_13; +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_13, 1); +x_21 = lean_ctor_get(x_13, 0); +lean_dec(x_21); +lean_inc(x_3); +x_22 = lean_array_to_list(x_3); +x_23 = lean_box(0); +x_24 = l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(x_22, x_23); +x_25 = l_Lean_MessageData_ofList(x_24); +x_26 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__2; +lean_ctor_set_tag(x_13, 7); +lean_ctor_set(x_13, 1, x_25); +lean_ctor_set(x_13, 0, x_26); +x_27 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__4; +x_28 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_28, 0, x_13); +lean_ctor_set(x_28, 1, x_27); +lean_inc(x_4); +x_29 = l_Lean_MessageData_ofExpr(x_4); +x_30 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +x_31 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +x_32 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_31); +x_33 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_12, x_32, x_5, x_6, x_7, x_8, x_9, x_10, 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); +x_36 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__5(x_1, x_3, x_4, x_2, x_34, x_5, x_6, x_7, x_8, x_9, x_10, x_35); +lean_dec(x_34); +return x_36; } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_23 = lean_ctor_get(x_13, 1); -lean_inc(x_23); +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_37 = lean_ctor_get(x_13, 1); +lean_inc(x_37); lean_dec(x_13); -x_24 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_24, 0, x_3); -lean_ctor_set(x_24, 1, x_4); -x_25 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_25, 0, x_24); -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_26, 1, x_23); -return x_26; +lean_inc(x_3); +x_38 = lean_array_to_list(x_3); +x_39 = lean_box(0); +x_40 = l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(x_38, x_39); +x_41 = l_Lean_MessageData_ofList(x_40); +x_42 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__2; +x_43 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_43, 0, x_42); +lean_ctor_set(x_43, 1, x_41); +x_44 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__4; +x_45 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_45, 0, x_43); +lean_ctor_set(x_45, 1, x_44); +lean_inc(x_4); +x_46 = l_Lean_MessageData_ofExpr(x_4); +x_47 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_47, 0, x_45); +lean_ctor_set(x_47, 1, x_46); +x_48 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +x_49 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_49, 0, x_47); +lean_ctor_set(x_49, 1, x_48); +x_50 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_12, x_49, x_5, x_6, x_7, x_8, x_9, x_10, x_37); +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_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__5(x_1, x_3, x_4, x_2, x_51, x_5, x_6, x_7, x_8, x_9, x_10, x_52); +lean_dec(x_51); +return x_53; } } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___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_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_11; uint8_t x_12; -x_11 = l_Lean_LocalDecl_userName(x_1); -x_12 = l_Lean_Name_hasMacroScopes(x_11); -lean_dec(x_11); -if (x_12 == 0) -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; -lean_dec(x_2); -lean_dec(x_1); -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_3); -lean_ctor_set(x_13, 1, x_4); -x_14 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_14, 0, x_13); -x_15 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_15, 0, x_14); -lean_ctor_set(x_15, 1, x_10); -return x_15; -} -else -{ -lean_object* x_16; lean_object* x_17; -x_16 = lean_box(0); -x_17 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__4(x_1, x_2, x_3, x_4, x_16, x_6, x_7, x_8, x_9, x_10); -return x_17; -} -} -} -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +lean_object* x_11; +x_11 = lean_ctor_get(x_1, 7); +lean_inc(x_11); +if (lean_obj_tag(x_11) == 0) { -lean_object* x_10; +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; uint8_t x_17; lean_object* x_18; +x_12 = l_Lean_Meta_mkFreshLevelMVar(x_6, x_7, x_8, x_9, x_10); +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_12, 1); +lean_inc(x_14); +lean_dec(x_12); +x_15 = l_Lean_Expr_sort___override(x_13); +x_16 = 1; +x_17 = 0; +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); lean_inc(x_5); -x_10 = l_Lean_Meta_getFVarLocalDecl(x_1, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_10) == 0) -{ -uint8_t x_11; -x_11 = !lean_is_exclusive(x_10); -if (x_11 == 0) -{ -lean_object* x_12; lean_object* x_13; uint8_t x_14; uint8_t x_15; -x_12 = lean_ctor_get(x_10, 0); -x_13 = lean_ctor_get(x_10, 1); -x_14 = l_Lean_LocalDecl_binderInfo(x_12); -x_15 = l_Lean_BinderInfo_isExplicit(x_14); -if (x_15 == 0) +lean_inc(x_4); +x_18 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_16, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_14); +if (lean_obj_tag(x_18) == 0) { -lean_object* x_16; lean_object* x_17; -lean_free_object(x_10); -x_16 = lean_box(0); -x_17 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__5(x_12, x_1, x_2, x_3, x_16, x_5, x_6, x_7, x_8, x_13); -lean_dec(x_5); -return x_17; +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 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__2___boxed), 11, 2); +lean_closure_set(x_20, 0, x_1); +lean_closure_set(x_20, 1, x_2); +x_21 = l_Lean_Elab_Term_addAutoBoundImplicits_x27___rarg(x_3, x_15, x_20, x_4, x_5, x_6, x_7, x_8, x_9, x_19); +return x_21; } else { -lean_object* x_18; lean_object* x_19; -lean_dec(x_12); +uint8_t x_22; +lean_dec(x_15); +lean_dec(x_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_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_2); -lean_ctor_set(x_18, 1, x_3); -x_19 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_19, 0, x_18); -lean_ctor_set(x_10, 0, x_19); -return x_10; -} +x_22 = !lean_is_exclusive(x_18); +if (x_22 == 0) +{ +return x_18; } else { -lean_object* x_20; lean_object* x_21; uint8_t x_22; uint8_t x_23; -x_20 = lean_ctor_get(x_10, 0); -x_21 = lean_ctor_get(x_10, 1); -lean_inc(x_21); -lean_inc(x_20); -lean_dec(x_10); -x_22 = l_Lean_LocalDecl_binderInfo(x_20); -x_23 = l_Lean_BinderInfo_isExplicit(x_22); -if (x_23 == 0) -{ -lean_object* x_24; lean_object* x_25; -x_24 = lean_box(0); -x_25 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__5(x_20, x_1, x_2, x_3, x_24, x_5, x_6, x_7, x_8, x_21); -lean_dec(x_5); +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_18, 0); +x_24 = lean_ctor_get(x_18, 1); +lean_inc(x_24); +lean_inc(x_23); +lean_dec(x_18); +x_25 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); return x_25; } +} +} else { lean_object* x_26; lean_object* x_27; lean_object* x_28; -lean_dec(x_20); -lean_dec(x_5); -lean_dec(x_1); -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_2); -lean_ctor_set(x_26, 1, x_3); -x_27 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_27, 0, 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_21); -return x_28; -} -} +x_26 = lean_ctor_get(x_11, 0); +lean_inc(x_26); +lean_dec(x_11); +x_27 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__4), 8, 1); +lean_closure_set(x_27, 0, x_26); +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_28 = l_Lean_Elab_Term_withAutoBoundImplicit___rarg(x_27, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_28) == 0) +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_29 = lean_ctor_get(x_28, 0); +lean_inc(x_29); +x_30 = lean_ctor_get(x_28, 1); +lean_inc(x_30); +lean_dec(x_28); +x_31 = lean_ctor_get(x_29, 0); +lean_inc(x_31); +lean_dec(x_29); +x_32 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___boxed), 11, 2); +lean_closure_set(x_32, 0, x_1); +lean_closure_set(x_32, 1, x_2); +x_33 = l_Lean_Elab_Term_addAutoBoundImplicits_x27___rarg(x_3, x_31, x_32, x_4, x_5, x_6, x_7, x_8, x_9, x_30); +return x_33; } else { -uint8_t x_29; +uint8_t x_34; +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_4); lean_dec(x_2); lean_dec(x_1); -x_29 = !lean_is_exclusive(x_10); -if (x_29 == 0) +x_34 = !lean_is_exclusive(x_28); +if (x_34 == 0) { -return x_10; +return x_28; } else { -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_dec(x_10); -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_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_28, 0); +x_36 = lean_ctor_get(x_28, 1); +lean_inc(x_36); +lean_inc(x_35); +lean_dec(x_28); +x_37 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +return x_37; } } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___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_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -uint8_t x_10; -x_10 = lean_usize_dec_lt(x_3, x_2); -if (x_10 == 0) -{ lean_object* x_11; -lean_dec(x_5); -x_11 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_11, 0, x_4); -lean_ctor_set(x_11, 1, x_9); -return x_11; -} -else -{ -lean_object* x_12; uint8_t x_13; -x_12 = lean_array_uget(x_1, x_3); -x_13 = !lean_is_exclusive(x_4); -if (x_13 == 0) -{ -lean_object* x_14; lean_object* x_15; uint8_t x_16; -x_14 = lean_ctor_get(x_4, 0); -x_15 = lean_ctor_get(x_4, 1); -x_16 = l_Lean_Expr_isFVar(x_12); -if (x_16 == 0) -{ -lean_object* x_17; -lean_dec(x_12); -lean_dec(x_5); -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_4); -lean_ctor_set(x_17, 1, x_9); -return x_17; -} -else -{ -uint8_t x_18; -x_18 = l_Array_contains___at_Lean_Meta_setMVarUserNamesAt___spec__1(x_14, x_12); -if (x_18 == 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_11 = l_Lean_Elab_Term_withAutoBoundImplicit___rarg(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_11) == 0) { -lean_object* x_19; -lean_dec(x_12); -lean_dec(x_5); -x_19 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_19, 0, x_4); -lean_ctor_set(x_19, 1, x_9); -return x_19; +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_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 = lean_nat_add(x_2, x_14); +x_16 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux(x_3, x_15, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +return x_16; } else { -lean_object* x_20; lean_object* x_21; -lean_free_object(x_4); -x_20 = lean_box(0); -lean_inc(x_5); -x_21 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__6(x_12, x_14, x_15, x_20, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_21) == 0) -{ -lean_object* x_22; -x_22 = lean_ctor_get(x_21, 0); -lean_inc(x_22); -if (lean_obj_tag(x_22) == 0) -{ -uint8_t x_23; +uint8_t x_17; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); lean_dec(x_5); -x_23 = !lean_is_exclusive(x_21); -if (x_23 == 0) +lean_dec(x_4); +lean_dec(x_3); +x_17 = !lean_is_exclusive(x_11); +if (x_17 == 0) { -lean_object* x_24; lean_object* x_25; -x_24 = lean_ctor_get(x_21, 0); -lean_dec(x_24); -x_25 = lean_ctor_get(x_22, 0); -lean_inc(x_25); -lean_dec(x_22); -lean_ctor_set(x_21, 0, x_25); -return x_21; +return x_11; } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_21, 1); -lean_inc(x_26); -lean_dec(x_21); -x_27 = lean_ctor_get(x_22, 0); -lean_inc(x_27); -lean_dec(x_22); -x_28 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_28, 0, x_27); -lean_ctor_set(x_28, 1, x_26); -return x_28; +lean_object* x_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; } } -else -{ -lean_object* x_29; lean_object* x_30; size_t x_31; size_t x_32; -x_29 = lean_ctor_get(x_21, 1); -lean_inc(x_29); -lean_dec(x_21); -x_30 = lean_ctor_get(x_22, 0); -lean_inc(x_30); -lean_dec(x_22); -x_31 = 1; -x_32 = lean_usize_add(x_3, x_31); -x_3 = x_32; -x_4 = x_30; -x_9 = x_29; -goto _start; } } -else +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_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_34; -lean_dec(x_5); -x_34 = !lean_is_exclusive(x_21); -if (x_34 == 0) +lean_object* x_11; lean_object* x_12; uint8_t x_13; +lean_inc(x_1); +x_11 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__1___boxed), 2, 1); +lean_closure_set(x_11, 0, x_1); +x_12 = lean_array_get_size(x_1); +x_13 = lean_nat_dec_lt(x_2, x_12); +lean_dec(x_12); +if (x_13 == 0) { -return x_21; +lean_object* x_14; lean_object* x_15; +lean_dec(x_2); +lean_dec(x_1); +x_14 = lean_alloc_closure((void*)(l_ReaderT_pure___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__12___rarg___boxed), 8, 1); +lean_closure_set(x_14, 0, x_3); +x_15 = l_Lean_Elab_Term_withAutoBoundImplicitForbiddenPred___rarg(x_11, x_14, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_15; } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_35 = lean_ctor_get(x_21, 0); -x_36 = lean_ctor_get(x_21, 1); -lean_inc(x_36); -lean_inc(x_35); -lean_dec(x_21); -x_37 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -return x_37; -} -} +lean_object* x_16; 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_array_fget(x_1, x_2); +x_17 = lean_ctor_get(x_16, 6); +lean_inc(x_17); +x_18 = l_Lean_Syntax_getArgs(x_17); +lean_dec(x_17); +x_19 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__7___boxed), 10, 2); +lean_closure_set(x_19, 0, x_16); +lean_closure_set(x_19, 1, x_3); +x_20 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabBinders___rarg), 9, 2); +lean_closure_set(x_20, 0, x_18); +lean_closure_set(x_20, 1, x_19); +x_21 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__8___boxed), 10, 3); +lean_closure_set(x_21, 0, x_20); +lean_closure_set(x_21, 1, x_2); +lean_closure_set(x_21, 2, x_1); +x_22 = l_Lean_Elab_Term_withAutoBoundImplicitForbiddenPred___rarg(x_11, x_21, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_22; } } } -else +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: { -lean_object* x_38; lean_object* x_39; uint8_t x_40; -x_38 = lean_ctor_get(x_4, 0); -x_39 = lean_ctor_get(x_4, 1); -lean_inc(x_39); -lean_inc(x_38); +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_40 = l_Lean_Expr_isFVar(x_12); -if (x_40 == 0) -{ -lean_object* x_41; lean_object* x_42; -lean_dec(x_12); -lean_dec(x_5); -x_41 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_41, 0, x_38); -lean_ctor_set(x_41, 1, x_39); -x_42 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_42, 0, x_41); -lean_ctor_set(x_42, 1, x_9); -return x_42; +x_7 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___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; } -else -{ -uint8_t x_43; -x_43 = l_Array_contains___at_Lean_Meta_setMVarUserNamesAt___spec__1(x_38, x_12); -if (x_43 == 0) -{ -lean_object* x_44; lean_object* x_45; -lean_dec(x_12); -lean_dec(x_5); -x_44 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_44, 0, x_38); -lean_ctor_set(x_44, 1, x_39); -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; } -else -{ -lean_object* x_46; lean_object* x_47; -x_46 = lean_box(0); -lean_inc(x_5); -x_47 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__6(x_12, x_38, x_39, x_46, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_47) == 0) +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { +_start: { -lean_object* x_48; -x_48 = lean_ctor_get(x_47, 0); -lean_inc(x_48); -if (lean_obj_tag(x_48) == 0) +uint8_t x_3; lean_object* x_4; +x_3 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: { -lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +lean_object* x_12; +x_12 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); lean_dec(x_5); -x_49 = lean_ctor_get(x_47, 1); -lean_inc(x_49); -if (lean_is_exclusive(x_47)) { - lean_ctor_release(x_47, 0); - lean_ctor_release(x_47, 1); - x_50 = x_47; -} else { - lean_dec_ref(x_47); - x_50 = lean_box(0); -} -x_51 = lean_ctor_get(x_48, 0); -lean_inc(x_51); -lean_dec(x_48); -if (lean_is_scalar(x_50)) { - x_52 = lean_alloc_ctor(0, 2, 0); -} else { - x_52 = x_50; +return x_12; } -lean_ctor_set(x_52, 0, x_51); -lean_ctor_set(x_52, 1, x_49); -return x_52; } -else +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: { -lean_object* x_53; lean_object* x_54; size_t x_55; size_t x_56; -x_53 = lean_ctor_get(x_47, 1); -lean_inc(x_53); -lean_dec(x_47); -x_54 = lean_ctor_get(x_48, 0); -lean_inc(x_54); -lean_dec(x_48); -x_55 = 1; -x_56 = lean_usize_add(x_3, x_55); -x_3 = x_56; -x_4 = x_54; -x_9 = x_53; -goto _start; +lean_object* x_10; +x_10 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__3(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; } } -else +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: { -lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; +lean_object* x_13; +x_13 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___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); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); lean_dec(x_5); -x_58 = lean_ctor_get(x_47, 0); -lean_inc(x_58); -x_59 = lean_ctor_get(x_47, 1); -lean_inc(x_59); -if (lean_is_exclusive(x_47)) { - lean_ctor_release(x_47, 0); - lean_ctor_release(x_47, 1); - x_60 = x_47; -} else { - lean_dec_ref(x_47); - x_60 = lean_box(0); +return x_13; } -if (lean_is_scalar(x_60)) { - x_61 = lean_alloc_ctor(1, 2, 0); -} else { - x_61 = x_60; } -lean_ctor_set(x_61, 0, x_58); -lean_ctor_set(x_61, 1, x_59); -return x_61; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +x_12 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +return x_12; } } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__7(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_3); +return x_11; +} } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_2); +return x_11; } } +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams___spec__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("invalid inductive type, number of parameters mismatch in mutually inductive datatypes", 85, 85); +return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___lambda__1___closed__1() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams___spec__1___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); +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams___spec__1___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams___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: { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; size_t x_18; size_t x_19; lean_object* x_20; -x_9 = lean_unsigned_to_nat(0u); -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); -x_13 = lean_unsigned_to_nat(1u); -x_14 = lean_nat_sub(x_10, x_13); +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_inc(x_3); -x_15 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_3, x_12, x_14); -x_16 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__3___closed__1; -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_2); -lean_ctor_set(x_17, 1, x_16); -x_18 = lean_array_size(x_15); -x_19 = 0; -lean_inc(x_4); -x_20 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4(x_15, x_18, x_19, x_17, x_4, x_5, x_6, x_7, 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; uint8_t x_18; +lean_dec(x_5); +x_15 = lean_array_uget(x_2, x_4); +x_16 = lean_ctor_get(x_15, 4); +lean_inc(x_16); +x_17 = lean_array_get_size(x_16); +lean_dec(x_16); +x_18 = lean_nat_dec_eq(x_17, x_1); +lean_dec(x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_19 = lean_ctor_get(x_15, 0); +lean_inc(x_19); lean_dec(x_15); -if (lean_obj_tag(x_20) == 0) +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +lean_dec(x_19); +x_21 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams___spec__1___closed__2; +x_22 = l_Lean_throwErrorAt___at_Lean_Elab_Term_Quotation_getAntiquotationIds___spec__1(x_20, x_21, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_20); +x_23 = !lean_is_exclusive(x_22); +if (x_23 == 0) { -uint8_t x_21; -x_21 = !lean_is_exclusive(x_20); -if (x_21 == 0) +return x_22; +} +else { -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; -x_22 = lean_ctor_get(x_20, 0); -x_23 = lean_ctor_get(x_20, 1); +lean_object* x_24; lean_object* x_25; lean_object* x_26; x_24 = lean_ctor_get(x_22, 0); -lean_inc(x_24); x_25 = lean_ctor_get(x_22, 1); lean_inc(x_25); +lean_inc(x_24); lean_dec(x_22); -x_26 = l_Array_isEmpty___rarg(x_25); -if (x_26 == 0) -{ -lean_object* x_27; uint8_t x_28; uint8_t x_29; uint8_t x_30; lean_object* x_31; -lean_free_object(x_20); -lean_dec(x_1); -lean_inc(x_25); -x_27 = l_Array_append___rarg(x_25, x_24); -lean_dec(x_24); -x_28 = 0; -x_29 = 1; -x_30 = 1; -lean_inc(x_3); -x_31 = l_Lean_Meta_mkForallFVars(x_27, x_3, x_28, x_29, x_30, x_4, x_5, x_6, x_7, 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; -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_Expr_getAppFn(x_3); -lean_dec(x_3); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -x_35 = lean_infer_type(x_34, x_4, x_5, x_6, x_7, x_33); -if (lean_obj_tag(x_35) == 0) -{ -lean_object* x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; -x_36 = lean_ctor_get(x_35, 0); -lean_inc(x_36); -x_37 = lean_ctor_get(x_35, 1); -lean_inc(x_37); -lean_dec(x_35); -x_38 = l_Lean_instantiateMVars___at___private_Lean_Meta_Basic_0__Lean_Meta_isClassApp_x3f___spec__1(x_36, x_4, x_5, x_6, x_7, x_37); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -x_39 = !lean_is_exclusive(x_38); -if (x_39 == 0) -{ -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_40 = lean_ctor_get(x_38, 0); -x_41 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getArrowBinderNames(x_40); -x_42 = lean_array_get_size(x_25); -lean_dec(x_25); -x_43 = l_Array_toSubarray___rarg(x_41, x_9, x_42); -x_44 = l_Array_ofSubarray___rarg(x_43); -lean_dec(x_43); -x_45 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceArrowBinderNames_go(x_44, x_32, x_9); -lean_dec(x_44); -lean_ctor_set(x_38, 0, x_45); -return x_38; -} -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; -x_46 = lean_ctor_get(x_38, 0); -x_47 = lean_ctor_get(x_38, 1); -lean_inc(x_47); -lean_inc(x_46); -lean_dec(x_38); -x_48 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getArrowBinderNames(x_46); -x_49 = lean_array_get_size(x_25); -lean_dec(x_25); -x_50 = l_Array_toSubarray___rarg(x_48, x_9, x_49); -x_51 = l_Array_ofSubarray___rarg(x_50); -lean_dec(x_50); -x_52 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceArrowBinderNames_go(x_51, x_32, x_9); -lean_dec(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; +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_54; -lean_dec(x_32); -lean_dec(x_25); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -x_54 = !lean_is_exclusive(x_35); -if (x_54 == 0) -{ -return x_35; +size_t x_27; size_t x_28; lean_object* x_29; +lean_dec(x_15); +x_27 = 1; +x_28 = lean_usize_add(x_4, x_27); +x_29 = lean_box(0); +x_4 = x_28; +x_5 = x_29; +goto _start; } -else -{ -lean_object* x_55; lean_object* x_56; lean_object* x_57; -x_55 = lean_ctor_get(x_35, 0); -x_56 = lean_ctor_get(x_35, 1); -lean_inc(x_56); -lean_inc(x_55); -lean_dec(x_35); -x_57 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_57, 0, x_55); -lean_ctor_set(x_57, 1, x_56); -return x_57; } } } -else -{ -uint8_t x_58; -lean_dec(x_25); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_58 = !lean_is_exclusive(x_31); -if (x_58 == 0) +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams(lean_object* x_1, lean_object* x_2, lean_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_31; -} -else +lean_object* x_9; lean_object* x_10; uint8_t x_11; size_t x_12; size_t x_13; lean_object* x_14; +x_9 = lean_array_get_size(x_1); +x_10 = lean_unsigned_to_nat(0u); +x_11 = lean_nat_dec_lt(x_10, x_9); +lean_dec(x_9); +x_12 = lean_array_size(x_1); +x_13 = 0; +if (x_11 == 0) { -lean_object* x_59; lean_object* x_60; lean_object* x_61; -x_59 = lean_ctor_get(x_31, 0); -x_60 = lean_ctor_get(x_31, 1); -lean_inc(x_60); -lean_inc(x_59); -lean_dec(x_31); -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_28; lean_object* x_29; +x_28 = l_Lean_Elab_Command_instInhabitedElabHeaderResult; +x_29 = l_outOfBounds___rarg(x_28); +x_14 = x_29; +goto block_27; } else { -lean_dec(x_25); -lean_dec(x_24); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_ctor_set(x_20, 0, x_1); -return x_20; -} +lean_object* x_30; +x_30 = lean_array_fget(x_1, x_10); +x_14 = x_30; +goto block_27; } -else -{ -lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; uint8_t x_66; -x_62 = lean_ctor_get(x_20, 0); -x_63 = lean_ctor_get(x_20, 1); -lean_inc(x_63); -lean_inc(x_62); -lean_dec(x_20); -x_64 = lean_ctor_get(x_62, 0); -lean_inc(x_64); -x_65 = lean_ctor_get(x_62, 1); -lean_inc(x_65); -lean_dec(x_62); -x_66 = l_Array_isEmpty___rarg(x_65); -if (x_66 == 0) -{ -lean_object* x_67; uint8_t x_68; uint8_t x_69; uint8_t x_70; lean_object* x_71; -lean_dec(x_1); -lean_inc(x_65); -x_67 = l_Array_append___rarg(x_65, x_64); -lean_dec(x_64); -x_68 = 0; -x_69 = 1; -x_70 = 1; -lean_inc(x_3); -x_71 = l_Lean_Meta_mkForallFVars(x_67, x_3, x_68, x_69, x_70, x_4, x_5, x_6, x_7, x_63); -if (lean_obj_tag(x_71) == 0) -{ -lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; -x_72 = lean_ctor_get(x_71, 0); -lean_inc(x_72); -x_73 = lean_ctor_get(x_71, 1); -lean_inc(x_73); -lean_dec(x_71); -x_74 = l_Lean_Expr_getAppFn(x_3); -lean_dec(x_3); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -x_75 = lean_infer_type(x_74, x_4, x_5, x_6, x_7, x_73); -if (lean_obj_tag(x_75) == 0) +block_27: { -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_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_instantiateMVars___at___private_Lean_Meta_Basic_0__Lean_Meta_isClassApp_x3f___spec__1(x_76, x_4, x_5, x_6, x_7, x_77); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -x_79 = lean_ctor_get(x_78, 0); -lean_inc(x_79); -x_80 = lean_ctor_get(x_78, 1); -lean_inc(x_80); -if (lean_is_exclusive(x_78)) { - lean_ctor_release(x_78, 0); - lean_ctor_release(x_78, 1); - x_81 = x_78; -} else { - lean_dec_ref(x_78); - x_81 = lean_box(0); -} -x_82 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getArrowBinderNames(x_79); -x_83 = lean_array_get_size(x_65); -lean_dec(x_65); -x_84 = l_Array_toSubarray___rarg(x_82, x_9, x_83); -x_85 = l_Array_ofSubarray___rarg(x_84); -lean_dec(x_84); -x_86 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceArrowBinderNames_go(x_85, x_72, x_9); -lean_dec(x_85); -if (lean_is_scalar(x_81)) { - x_87 = lean_alloc_ctor(0, 2, 0); -} else { - x_87 = x_81; -} -lean_ctor_set(x_87, 0, x_86); -lean_ctor_set(x_87, 1, x_80); -return x_87; -} -else +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_15 = lean_ctor_get(x_14, 4); +lean_inc(x_15); +lean_dec(x_14); +x_16 = lean_array_get_size(x_15); +lean_dec(x_15); +x_17 = lean_box(0); +x_18 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams___spec__1(x_16, x_1, x_12, x_13, x_17, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_18) == 0) { -lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; -lean_dec(x_72); -lean_dec(x_65); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -x_88 = lean_ctor_get(x_75, 0); -lean_inc(x_88); -x_89 = lean_ctor_get(x_75, 1); -lean_inc(x_89); -if (lean_is_exclusive(x_75)) { - lean_ctor_release(x_75, 0); - lean_ctor_release(x_75, 1); - x_90 = x_75; -} else { - lean_dec_ref(x_75); - x_90 = lean_box(0); -} -if (lean_is_scalar(x_90)) { - x_91 = lean_alloc_ctor(1, 2, 0); -} else { - x_91 = x_90; -} -lean_ctor_set(x_91, 0, x_88); -lean_ctor_set(x_91, 1, x_89); -return x_91; -} -} -else +uint8_t x_19; +x_19 = !lean_is_exclusive(x_18); +if (x_19 == 0) { -lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; -lean_dec(x_65); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_92 = lean_ctor_get(x_71, 0); -lean_inc(x_92); -x_93 = lean_ctor_get(x_71, 1); -lean_inc(x_93); -if (lean_is_exclusive(x_71)) { - lean_ctor_release(x_71, 0); - lean_ctor_release(x_71, 1); - x_94 = x_71; -} else { - lean_dec_ref(x_71); - x_94 = lean_box(0); -} -if (lean_is_scalar(x_94)) { - x_95 = lean_alloc_ctor(1, 2, 0); -} else { - x_95 = x_94; -} -lean_ctor_set(x_95, 0, x_92); -lean_ctor_set(x_95, 1, x_93); -return x_95; -} +lean_object* x_20; +x_20 = lean_ctor_get(x_18, 0); +lean_dec(x_20); +lean_ctor_set(x_18, 0, x_16); +return x_18; } else { -lean_object* x_96; -lean_dec(x_65); -lean_dec(x_64); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_96 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_96, 0, x_1); -lean_ctor_set(x_96, 1, x_63); -return x_96; -} +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_16); +lean_ctor_set(x_22, 1, x_21); +return x_22; } } else { -uint8_t x_97; -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_97 = !lean_is_exclusive(x_20); -if (x_97 == 0) +uint8_t x_23; +lean_dec(x_16); +x_23 = !lean_is_exclusive(x_18); +if (x_23 == 0) { -return x_20; +return x_18; } else { -lean_object* x_98; lean_object* x_99; lean_object* x_100; -x_98 = lean_ctor_get(x_20, 0); -x_99 = lean_ctor_get(x_20, 1); -lean_inc(x_99); -lean_inc(x_98); -lean_dec(x_20); -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_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_18, 0); +x_25 = lean_ctor_get(x_18, 1); +lean_inc(x_25); +lean_inc(x_24); +lean_dec(x_18); +x_26 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_26, 0, x_24); +lean_ctor_set(x_26, 1, x_25); +return x_26; } } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs(lean_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_inc(x_1); -x_7 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___lambda__1), 8, 1); -lean_closure_set(x_7, 0, x_1); -x_8 = 0; -x_9 = l_Lean_Meta_forallTelescopeReducing___at_Lean_Meta_getParamNames___spec__2___rarg(x_1, x_7, x_8, x_2, x_3, x_4, x_5, x_6); -return x_9; } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams___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_5; size_t x_6; uint8_t x_7; lean_object* x_8; -x_5 = lean_unbox_usize(x_3); +size_t x_13; size_t x_14; lean_object* x_15; +x_13 = lean_unbox_usize(x_3); lean_dec(x_3); -x_6 = lean_unbox_usize(x_4); +x_14 = lean_unbox_usize(x_4); lean_dec(x_4); -x_7 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__1(x_1, x_2, x_5, x_6); +x_15 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams___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_11); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_2); lean_dec(x_1); -x_8 = lean_box(x_7); -return x_8; +return x_15; } } -LEAN_EXPORT lean_object* l_Lean_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___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_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams___boxed(lean_object* x_1, lean_object* x_2, lean_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_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams(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); return x_9; } } -LEAN_EXPORT lean_object* l_Array_erase___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__3___boxed(lean_object* x_1, lean_object* x_2) { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe___spec__1___closed__1() { _start: { -lean_object* x_3; -x_3 = l_Array_erase___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__3(x_1, x_2); -lean_dec(x_2); -return x_3; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("invalid inductive type, cannot mix unsafe and safe declarations in a mutually inductive datatypes", 97, 97); +return x_1; } } -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* x_1, lean_object* x_2) { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe___spec__1___closed__2() { _start: { -uint8_t x_3; lean_object* x_4; -x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__1(x_1, x_2); -lean_dec(x_2); -lean_dec(x_1); -x_4 = lean_box(x_3); -return x_4; +lean_object* x_1; lean_object* x_2; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe___spec__1___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__2___boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe___spec__1(uint8_t 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_2; lean_object* x_3; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__2(x_1); -lean_dec(x_1); -x_3 = lean_box(x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +uint8_t x_13; +x_13 = lean_usize_dec_lt(x_4, x_3); +if (x_13 == 0) { -lean_object* x_10; -x_10 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_8); -lean_dec(x_7); +lean_object* x_14; +lean_dec(x_10); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -return x_10; -} +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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___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: +else { -lean_object* x_11; -x_11 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__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); -lean_dec(x_6); +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_26; uint8_t x_27; lean_dec(x_5); -return x_11; +x_15 = lean_array_uget(x_2, x_4); +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +lean_dec(x_15); +x_26 = lean_ctor_get(x_16, 2); +lean_inc(x_26); +x_27 = lean_ctor_get_uint8(x_26, sizeof(void*)*3 + 3); +lean_dec(x_26); +if (x_27 == 0) +{ +if (x_1 == 0) +{ +size_t x_28; size_t x_29; lean_object* x_30; +lean_dec(x_16); +x_28 = 1; +x_29 = lean_usize_add(x_4, x_28); +x_30 = lean_box(0); +x_4 = x_29; +x_5 = x_30; +goto _start; +} +else +{ +lean_object* x_32; +x_32 = lean_box(0); +x_17 = x_32; +goto block_25; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: +else { -lean_object* x_11; -x_11 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__5(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; -} +if (x_1 == 0) +{ +lean_object* x_33; +x_33 = lean_box(0); +x_17 = x_33; +goto block_25; } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +else { -lean_object* x_10; -x_10 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__6(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_4); -return x_10; +size_t x_34; size_t x_35; lean_object* x_36; +lean_dec(x_16); +x_34 = 1; +x_35 = lean_usize_add(x_4, x_34); +x_36 = lean_box(0); +x_4 = x_35; +x_5 = x_36; +goto _start; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___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) { -_start: +block_25: { -size_t x_10; size_t x_11; lean_object* x_12; -x_10 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_11 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_12 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4(x_1, x_10, x_11, 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_1); -return x_12; +lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +lean_dec(x_17); +x_18 = lean_ctor_get(x_16, 0); +lean_inc(x_18); +lean_dec(x_16); +x_19 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe___spec__1___closed__2; +x_20 = l_Lean_throwErrorAt___at_Lean_Elab_Term_Quotation_getAntiquotationIds___spec__1(x_18, x_19, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_18); +x_21 = !lean_is_exclusive(x_20); +if (x_21 == 0) +{ +return x_20; +} +else +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_20, 0); +x_23 = lean_ctor_get(x_20, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_20); +x_24 = lean_alloc_ctor(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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___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_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe(lean_object* x_1, lean_object* x_2, lean_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_12; -x_12 = lean_usize_dec_lt(x_3, x_2); -if (x_12 == 0) +lean_object* x_9; lean_object* x_10; uint8_t x_11; size_t x_12; size_t x_13; lean_object* x_14; +x_9 = lean_array_get_size(x_1); +x_10 = lean_unsigned_to_nat(0u); +x_11 = lean_nat_dec_lt(x_10, x_9); +lean_dec(x_9); +x_12 = lean_array_size(x_1); +x_13 = 0; +if (x_11 == 0) { -lean_object* x_13; -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; +lean_object* x_29; lean_object* x_30; +x_29 = l_Lean_Elab_Command_instInhabitedElabHeaderResult; +x_30 = l_outOfBounds___rarg(x_29); +x_14 = x_30; +goto block_28; } else { -lean_object* x_14; lean_object* x_15; -x_14 = lean_array_uget(x_1, x_3); -lean_inc(x_7); -x_15 = l_Lean_Meta_getFVarLocalDecl(x_14, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_15) == 0) +lean_object* x_31; +x_31 = lean_array_fget(x_1, x_10); +x_14 = x_31; +goto block_28; +} +block_28: { -lean_object* x_16; lean_object* x_17; uint8_t x_18; uint8_t x_19; -x_16 = lean_ctor_get(x_15, 0); +lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; lean_object* x_19; +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +lean_dec(x_14); +x_16 = lean_ctor_get(x_15, 2); lean_inc(x_16); -x_17 = lean_ctor_get(x_15, 1); -lean_inc(x_17); lean_dec(x_15); -x_18 = l_Lean_LocalDecl_binderInfo(x_16); +x_17 = lean_ctor_get_uint8(x_16, sizeof(void*)*3 + 3); lean_dec(x_16); -x_19 = l_Lean_BinderInfo_isExplicit(x_18); -if (x_19 == 0) +x_18 = lean_box(0); +x_19 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe___spec__1(x_17, x_1, x_12, x_13, x_18, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_19) == 0) { -size_t x_20; size_t x_21; -lean_dec(x_14); -x_20 = 1; -x_21 = lean_usize_add(x_3, x_20); -x_3 = x_21; -x_11 = x_17; -goto _start; +uint8_t x_20; +x_20 = !lean_is_exclusive(x_19); +if (x_20 == 0) +{ +lean_object* x_21; +x_21 = lean_ctor_get(x_19, 0); +lean_dec(x_21); +lean_ctor_set(x_19, 0, x_18); +return x_19; } else { -lean_object* x_23; uint8_t x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; size_t x_28; size_t x_29; -x_23 = l_Lean_Expr_fvarId_x21(x_14); -lean_dec(x_14); -x_24 = 1; -x_25 = lean_box(x_24); -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_27 = lean_array_push(x_4, x_26); -x_28 = 1; -x_29 = lean_usize_add(x_3, x_28); -x_3 = x_29; -x_4 = x_27; -x_11 = x_17; -goto _start; +lean_object* x_22; lean_object* x_23; +x_22 = lean_ctor_get(x_19, 1); +lean_inc(x_22); +lean_dec(x_19); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_18); +lean_ctor_set(x_23, 1, x_22); +return x_23; } } else { -uint8_t x_31; -lean_dec(x_14); -lean_dec(x_7); -lean_dec(x_4); -x_31 = !lean_is_exclusive(x_15); -if (x_31 == 0) +uint8_t x_24; +x_24 = !lean_is_exclusive(x_19); +if (x_24 == 0) { -return x_15; +return x_19; } else { -lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_32 = lean_ctor_get(x_15, 0); -x_33 = lean_ctor_get(x_15, 1); -lean_inc(x_33); -lean_inc(x_32); -lean_dec(x_15); -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_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_19, 0); +x_26 = lean_ctor_get(x_19, 1); +lean_inc(x_26); +lean_inc(x_25); +lean_dec(x_19); +x_27 = lean_alloc_ctor(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_Meta_withNewBinderInfos___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_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_withNewBinderInfosImp___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); +uint8_t x_13; size_t x_14; size_t x_15; lean_object* x_16; +x_13 = lean_unbox(x_1); +lean_dec(x_1); +x_14 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_15 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_16 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe___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_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_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_2); +return x_16; } -else -{ -uint8_t x_16; -x_16 = !lean_is_exclusive(x_11); -if (x_16 == 0) -{ -return x_11; } -else +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe___boxed(lean_object* x_1, lean_object* x_2, lean_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_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_9; +x_9 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +return x_9; } } +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_InductiveView_checkLevelNames___spec__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("invalid inductive type, universe parameters mismatch in mutually inductive datatypes", 84, 84); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Meta_withNewBinderInfos___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___spec__2(lean_object* x_1) { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_InductiveView_checkLevelNames___spec__1___closed__2() { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withNewBinderInfos___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___spec__2___rarg___boxed), 9, 0); +lean_object* x_1; lean_object* x_2; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_InductiveView_checkLevelNames___spec__1___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___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_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_InductiveView_checkLevelNames___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: { -size_t x_10; size_t x_11; lean_object* x_12; lean_object* x_13; -x_10 = lean_array_size(x_1); -x_11 = 0; -x_12 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__3___closed__1; -lean_inc(x_5); -x_13 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___spec__1(x_1, x_10, x_11, x_12, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_13) == 0) +uint8_t x_13; +x_13 = lean_usize_dec_lt(x_4, x_3); +if (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_Lean_Meta_withNewBinderInfos___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___spec__2___rarg(x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_15); -lean_dec(x_14); -return x_16; +lean_object* x_14; +lean_dec(x_10); +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 { -uint8_t x_17; -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); +lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_17 = !lean_is_exclusive(x_13); +x_15 = lean_array_uget(x_2, x_4); +x_16 = lean_ctor_get(x_15, 5); +lean_inc(x_16); +x_17 = l_List_beq___at___private_Lean_Declaration_0__Lean_beqConstantVal____x40_Lean_Declaration___hyg_433____spec__1(x_16, x_1); +lean_dec(x_16); if (x_17 == 0) { -return x_13; +lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_18 = lean_ctor_get(x_15, 0); +lean_inc(x_18); +lean_dec(x_15); +x_19 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_InductiveView_checkLevelNames___spec__1___closed__2; +x_20 = l_Lean_throwErrorAt___at_Lean_Elab_Term_Quotation_getAntiquotationIds___spec__1(x_18, x_19, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_18); +x_21 = !lean_is_exclusive(x_20); +if (x_21 == 0) +{ +return x_20; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_13, 0); -x_19 = lean_ctor_get(x_13, 1); -lean_inc(x_19); -lean_inc(x_18); -lean_dec(x_13); -x_20 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_20, 0, x_18); -lean_ctor_set(x_20, 1, x_19); -return x_20; +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_20, 0); +x_23 = lean_ctor_get(x_20, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_20); +x_24 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); +return x_24; } } +else +{ +size_t x_25; size_t x_26; lean_object* x_27; +lean_dec(x_15); +x_25 = 1; +x_26 = lean_usize_add(x_4, x_25); +x_27 = lean_box(0); +x_4 = x_26; +x_5 = x_27; +goto _start; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___rarg___boxed), 9, 0); -return x_2; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_InductiveView_checkLevelNames(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -size_t x_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_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___spec__1(x_1, x_12, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_10); +lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_9 = lean_array_get_size(x_1); +x_10 = lean_unsigned_to_nat(1u); +x_11 = lean_nat_dec_lt(x_10, x_9); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; lean_dec(x_9); -lean_dec(x_8); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_1); -return x_14; +lean_dec(x_2); +x_12 = lean_box(0); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_8); +return x_13; } +else +{ +lean_object* x_14; uint8_t x_15; size_t x_16; size_t x_17; lean_object* x_18; +x_14 = lean_unsigned_to_nat(0u); +x_15 = lean_nat_dec_lt(x_14, x_9); +lean_dec(x_9); +x_16 = lean_array_size(x_1); +x_17 = 0; +if (x_15 == 0) +{ +lean_object* x_31; lean_object* x_32; +x_31 = l_Lean_Elab_Command_instInhabitedInductiveView; +x_32 = l_outOfBounds___rarg(x_31); +x_18 = x_32; +goto block_30; } -LEAN_EXPORT lean_object* l_Lean_Meta_withNewBinderInfos___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___spec__2___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +else { -lean_object* x_10; -x_10 = l_Lean_Meta_withNewBinderInfos___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___spec__2___rarg(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_33; +x_33 = lean_array_fget(x_1, x_14); +x_18 = x_33; +goto block_30; } +block_30: +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_18, 5); +lean_inc(x_19); +lean_dec(x_18); +x_20 = lean_box(0); +x_21 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_InductiveView_checkLevelNames___spec__1(x_19, x_1, x_16, x_17, x_20, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_19); +if (lean_obj_tag(x_21) == 0) +{ +uint8_t x_22; +x_22 = !lean_is_exclusive(x_21); +if (x_22 == 0) +{ +lean_object* x_23; +x_23 = lean_ctor_get(x_21, 0); +lean_dec(x_23); +lean_ctor_set(x_21, 0, x_20); +return x_21; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___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) { -_start: +else { -lean_object* x_10; -x_10 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___rarg(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_24; lean_object* x_25; +x_24 = lean_ctor_get(x_21, 1); +lean_inc(x_24); +lean_dec(x_21); +x_25 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_25, 0, x_20); +lean_ctor_set(x_25, 1, x_24); +return x_25; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_10 = lean_array_set(x_3, x_1, x_2); -x_11 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_11, 0, 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; -} +uint8_t x_26; +x_26 = !lean_is_exclusive(x_21); +if (x_26 == 0) +{ +return x_21; } -static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___spec__1___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("inductive datatype parameter mismatch", 37, 37); -return x_1; +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_21, 0); +x_28 = lean_ctor_get(x_21, 1); +lean_inc(x_28); +lean_inc(x_27); +lean_dec(x_21); +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_27); +lean_ctor_set(x_29, 1, x_28); +return x_29; } } -static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___spec__1___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___spec__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_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___spec__1___closed__3() { +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_InductiveView_checkLevelNames___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("\nexpected", 9, 9); -return x_1; +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_Elab_Inductive_0__Lean_Elab_Command_InductiveView_checkLevelNames___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_11); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_2); +lean_dec(x_1); +return x_15; } } -static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___spec__1___closed__4() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_InductiveView_checkLevelNames___boxed(lean_object* x_1, lean_object* x_2, lean_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_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___spec__1___closed__3; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +lean_object* x_9; +x_9 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_InductiveView_checkLevelNames(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +return x_9; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_ElabHeaderResult_checkLevelNames___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; -x_13 = lean_nat_dec_le(x_5, x_4); +x_13 = lean_usize_dec_lt(x_4, x_3); if (x_13 == 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_14; +lean_dec(x_10); +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_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; uint8_t x_20; lean_object* x_21; -x_16 = lean_unsigned_to_nat(1u); -x_17 = lean_nat_sub(x_3, x_16); -lean_dec(x_3); -x_18 = lean_nat_dec_lt(x_4, x_2); -x_19 = lean_array_get_size(x_7); -x_20 = lean_nat_dec_lt(x_4, x_19); +lean_object* x_15; lean_object* x_16; uint8_t x_17; +lean_dec(x_5); +x_15 = lean_array_uget(x_2, x_4); +x_16 = lean_ctor_get(x_15, 3); +lean_inc(x_16); +x_17 = l_List_beq___at___private_Lean_Declaration_0__Lean_beqConstantVal____x40_Lean_Declaration___hyg_433____spec__1(x_16, x_1); +lean_dec(x_16); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; +x_18 = lean_ctor_get(x_15, 0); +lean_inc(x_18); +lean_dec(x_15); +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +lean_dec(x_18); +x_20 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_InductiveView_checkLevelNames___spec__1___closed__2; +x_21 = l_Lean_throwErrorAt___at_Lean_Elab_Term_Quotation_getAntiquotationIds___spec__1(x_19, x_20, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_19); -if (x_18 == 0) +x_22 = !lean_is_exclusive(x_21); +if (x_22 == 0) { -lean_object* x_58; lean_object* x_59; -x_58 = l_Lean_instInhabitedExpr; -x_59 = l_outOfBounds___rarg(x_58); -x_21 = x_59; -goto block_57; +return x_21; } else { -lean_object* x_60; -x_60 = lean_array_fget(x_1, x_4); -x_21 = x_60; -goto block_57; +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_21, 0); +x_24 = lean_ctor_get(x_21, 1); +lean_inc(x_24); +lean_inc(x_23); +lean_dec(x_21); +x_25 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +return x_25; } -block_57: -{ -lean_object* x_22; -if (x_20 == 0) -{ -lean_object* x_54; lean_object* x_55; -x_54 = l_Lean_instInhabitedExpr; -x_55 = l_outOfBounds___rarg(x_54); -x_22 = x_55; -goto block_53; } else { -lean_object* x_56; -x_56 = lean_array_fget(x_7, x_4); -x_22 = x_56; -goto block_53; +size_t x_26; size_t x_27; lean_object* x_28; +lean_dec(x_15); +x_26 = 1; +x_27 = lean_usize_add(x_4, x_26); +x_28 = lean_box(0); +x_4 = x_27; +x_5 = x_28; +goto _start; } -block_53: +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_ElabHeaderResult_checkLevelNames(lean_object* x_1, lean_object* x_2, lean_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_23; -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_22); -lean_inc(x_21); -x_23 = l_Lean_Meta_isExprDefEq(x_21, x_22, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_23) == 0) +lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_9 = lean_array_get_size(x_1); +x_10 = lean_unsigned_to_nat(1u); +x_11 = lean_nat_dec_lt(x_10, x_9); +if (x_11 == 0) { -lean_object* x_24; uint8_t x_25; -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -x_25 = lean_unbox(x_24); -lean_dec(x_24); -if (x_25 == 0) +lean_object* x_12; lean_object* x_13; +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_2); +x_12 = lean_box(0); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_8); +return x_13; +} +else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; -lean_dec(x_17); -lean_dec(x_7); -lean_dec(x_4); -x_26 = lean_ctor_get(x_23, 1); -lean_inc(x_26); -lean_dec(x_23); -x_27 = l_Lean_indentExpr(x_22); -x_28 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___spec__1___closed__2; -x_29 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_29, 0, x_28); -lean_ctor_set(x_29, 1, x_27); -x_30 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___spec__1___closed__4; -x_31 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_31, 0, x_29); -lean_ctor_set(x_31, 1, x_30); -x_32 = l_Lean_indentExpr(x_21); -x_33 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_33, 0, x_31); -lean_ctor_set(x_33, 1, x_32); -x_34 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5; -x_35 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_35, 0, x_33); -lean_ctor_set(x_35, 1, x_34); -x_36 = l_Lean_throwError___at_Lean_Meta_mkSimpCongrTheorem___spec__4(x_35, x_8, x_9, x_10, x_11, x_26); -lean_dec(x_11); -lean_dec(x_10); +lean_object* x_14; uint8_t x_15; size_t x_16; size_t x_17; lean_object* x_18; +x_14 = lean_unsigned_to_nat(0u); +x_15 = lean_nat_dec_lt(x_14, x_9); lean_dec(x_9); -lean_dec(x_8); -x_37 = !lean_is_exclusive(x_36); -if (x_37 == 0) +x_16 = lean_array_size(x_1); +x_17 = 0; +if (x_15 == 0) { -return x_36; +lean_object* x_31; lean_object* x_32; +x_31 = l_Lean_Elab_Command_instInhabitedElabHeaderResult; +x_32 = l_outOfBounds___rarg(x_31); +x_18 = x_32; +goto block_30; } 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_object* x_33; +x_33 = lean_array_fget(x_1, x_14); +x_18 = x_33; +goto block_30; } +block_30: +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_18, 3); +lean_inc(x_19); +lean_dec(x_18); +x_20 = lean_box(0); +x_21 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_ElabHeaderResult_checkLevelNames___spec__1(x_19, x_1, x_16, x_17, x_20, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_19); +if (lean_obj_tag(x_21) == 0) +{ +uint8_t x_22; +x_22 = !lean_is_exclusive(x_21); +if (x_22 == 0) +{ +lean_object* x_23; +x_23 = lean_ctor_get(x_21, 0); +lean_dec(x_23); +lean_ctor_set(x_21, 0, x_20); +return x_21; } else { -lean_object* x_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_22); -x_41 = lean_ctor_get(x_23, 1); -lean_inc(x_41); -lean_dec(x_23); -x_42 = lean_box(0); -x_43 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___spec__1___lambda__1(x_4, x_21, x_7, x_42, x_8, x_9, x_10, x_11, x_41); -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_ctor_get(x_44, 0); -lean_inc(x_46); -lean_dec(x_44); -x_47 = lean_nat_add(x_4, x_6); -lean_dec(x_4); -x_3 = x_17; -x_4 = x_47; -x_7 = x_46; -x_12 = x_45; -goto _start; +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_21, 1); +lean_inc(x_24); +lean_dec(x_21); +x_25 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_25, 0, x_20); +lean_ctor_set(x_25, 1, x_24); +return x_25; } } else { -uint8_t x_49; -lean_dec(x_22); -lean_dec(x_21); -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); -x_49 = !lean_is_exclusive(x_23); -if (x_49 == 0) +uint8_t x_26; +x_26 = !lean_is_exclusive(x_21); +if (x_26 == 0) { -return x_23; +return x_21; } else { -lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_50 = lean_ctor_get(x_23, 0); -x_51 = lean_ctor_get(x_23, 1); -lean_inc(x_51); -lean_inc(x_50); -lean_dec(x_23); -x_52 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_52, 0, x_50); -lean_ctor_set(x_52, 1, x_51); -return x_52; +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_21, 0); +x_28 = lean_ctor_get(x_21, 1); +lean_inc(x_28); +lean_inc(x_27); +lean_dec(x_21); +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_27); +lean_ctor_set(x_29, 1, x_28); +return x_29; } } } } } -else +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_ElabHeaderResult_checkLevelNames___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: { -lean_object* x_61; +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_Elab_Inductive_0__Lean_Elab_Command_ElabHeaderResult_checkLevelNames___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_11); -lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_2); +lean_dec(x_1); +return x_15; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_ElabHeaderResult_checkLevelNames___boxed(lean_object* x_1, lean_object* x_2, lean_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_Inductive_0__Lean_Elab_Command_ElabHeaderResult_checkLevelNames(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_7); +lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_61 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_61, 0, x_7); -lean_ctor_set(x_61, 1, x_12); -return x_61; +lean_dec(x_1); +return x_9; } } -else +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkTypeFor___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_62; -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); +uint8_t x_10; uint8_t x_11; uint8_t x_12; lean_object* x_13; +x_10 = 0; +x_11 = 1; +x_12 = 1; +x_13 = l_Lean_Meta_mkForallFVars(x_1, x_2, x_10, x_11, x_12, x_5, x_6, x_7, x_8, x_9); +return x_13; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkTypeFor(lean_object* x_1, lean_object* x_2, lean_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_ctor_get(x_1, 1); +lean_inc(x_9); +x_10 = lean_ctor_get(x_1, 2); +lean_inc(x_10); +x_11 = lean_ctor_get(x_1, 4); +lean_inc(x_11); +x_12 = lean_ctor_get(x_1, 5); +lean_inc(x_12); +lean_dec(x_1); +x_13 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkTypeFor___lambda__1___boxed), 9, 2); +lean_closure_set(x_13, 0, x_11); +lean_closure_set(x_13, 1, x_12); +x_14 = l_Lean_Meta_withLCtx___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__3___rarg(x_9, x_10, x_13, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +return x_14; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkTypeFor___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkTypeFor___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_62 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_62, 0, x_7); -lean_ctor_set(x_62, 1, x_12); -return x_62; -} +return x_10; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___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; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_10 = lean_array_get_size(x_1); -x_11 = lean_unsigned_to_nat(0u); -x_12 = lean_unsigned_to_nat(1u); +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_6, 5); +x_10 = lean_ctor_get(x_2, 2); lean_inc(x_10); -x_13 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___spec__1(x_1, x_10, x_10, x_11, x_10, x_12, x_3, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_10); -if (lean_obj_tag(x_13) == 0) +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_is_exclusive(x_12); +if (x_13 == 0) { -uint8_t x_14; -x_14 = !lean_is_exclusive(x_13); -if (x_14 == 0) +lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_14 = lean_ctor_get(x_12, 0); +x_15 = lean_ctor_get(x_12, 1); +x_16 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(x_14, x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_15); +lean_dec(x_2); +x_17 = !lean_is_exclusive(x_16); +if (x_17 == 0) { -lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = lean_ctor_get(x_13, 0); -x_16 = l_Lean_mkAppN(x_2, x_15); -lean_dec(x_15); -x_17 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_17, 0, x_16); -lean_ctor_set(x_13, 0, x_17); -return x_13; +lean_object* x_18; +x_18 = lean_ctor_get(x_16, 0); +lean_ctor_set(x_12, 1, x_18); +lean_ctor_set(x_12, 0, x_11); +lean_ctor_set_tag(x_16, 1); +lean_ctor_set(x_16, 0, x_12); +return x_16; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_18 = lean_ctor_get(x_13, 0); -x_19 = lean_ctor_get(x_13, 1); +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_16, 0); +x_20 = lean_ctor_get(x_16, 1); +lean_inc(x_20); lean_inc(x_19); -lean_inc(x_18); -lean_dec(x_13); -x_20 = l_Lean_mkAppN(x_2, x_18); -lean_dec(x_18); -x_21 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_21, 0, x_20); -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_21); -lean_ctor_set(x_22, 1, x_19); -return x_22; +lean_dec(x_16); +lean_ctor_set(x_12, 1, x_19); +lean_ctor_set(x_12, 0, x_11); +x_21 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_21, 0, x_12); +lean_ctor_set(x_21, 1, x_20); +return x_21; } } else { -uint8_t x_23; +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_22 = lean_ctor_get(x_12, 0); +x_23 = lean_ctor_get(x_12, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_12); +x_24 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(x_22, x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_23); lean_dec(x_2); -x_23 = !lean_is_exclusive(x_13); -if (x_23 == 0) -{ -return x_13; -} -else -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_13, 0); -x_25 = lean_ctor_get(x_13, 1); +x_25 = lean_ctor_get(x_24, 0); lean_inc(x_25); -lean_inc(x_24); -lean_dec(x_13); -x_26 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_26, 0, x_24); -lean_ctor_set(x_26, 1, x_25); -return x_26; +x_26 = lean_ctor_get(x_24, 1); +lean_inc(x_26); +if (lean_is_exclusive(x_24)) { + lean_ctor_release(x_24, 0); + lean_ctor_release(x_24, 1); + x_27 = x_24; +} else { + lean_dec_ref(x_24); + x_27 = lean_box(0); +} +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_11); +lean_ctor_set(x_28, 1, x_25); +if (lean_is_scalar(x_27)) { + x_29 = lean_alloc_ctor(1, 2, 0); +} else { + x_29 = x_27; + lean_ctor_set_tag(x_29, 1); } +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_26); +return x_29; } } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___lambda__2___closed__1() { +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___spec__1(lean_object* x_1) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = lean_box(0); -x_2 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_2, 0, x_1); +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___spec__1___rarg___boxed), 8, 0); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___lambda__2___closed__2() { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___rarg___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("unexpected inductive type occurrence", 36, 36); +x_1 = lean_mk_string_unchecked("unexpected inductive resulting type", 35, 35); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___lambda__2___closed__3() { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___rarg___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___lambda__2___closed__2; +x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___rarg___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___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_9; uint8_t x_10; -x_9 = l_Lean_Expr_getAppFn(x_3); -x_10 = l_Array_contains___at_Lean_Meta_setMVarUserNamesAt___spec__1(x_1, x_9); -if (x_10 == 0) +lean_object* x_8; lean_object* x_9; +x_8 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___rarg___closed__2; +x_9 = l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___spec__1___rarg(x_8, x_1, x_2, x_3, x_4, x_5, x_6, x_7); +return x_9; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType(lean_object* x_1) { +_start: { -lean_object* x_11; lean_object* x_12; -lean_dec(x_9); +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___rarg___boxed), 7, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +x_9 = l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___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); -x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___lambda__2___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_8); -return x_12; +return x_9; } -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___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); -x_17 = lean_unsigned_to_nat(1u); -x_18 = lean_nat_sub(x_14, x_17); -lean_dec(x_14); -lean_inc(x_3); -x_19 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_3, x_16, x_18); -x_20 = lean_array_get_size(x_2); -x_21 = lean_array_get_size(x_19); -x_22 = lean_nat_dec_le(x_20, x_21); -lean_dec(x_21); -lean_dec(x_20); -if (x_22 == 0) +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___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_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_dec(x_9); -x_23 = l_Lean_indentExpr(x_3); -x_24 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___lambda__2___closed__3; -x_25 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_25, 0, x_24); -lean_ctor_set(x_25, 1, x_23); -x_26 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5; -x_27 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_26); -x_28 = l_Lean_throwError___at_Lean_Meta_mkSimpCongrTheorem___spec__4(x_27, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_7); +lean_object* x_8; +x_8 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_29 = !lean_is_exclusive(x_28); -if (x_29 == 0) -{ -return x_28; -} -else -{ -lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_30 = lean_ctor_get(x_28, 0); -x_31 = lean_ctor_get(x_28, 1); -lean_inc(x_31); -lean_inc(x_30); -lean_dec(x_28); -x_32 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_32, 0, x_30); -lean_ctor_set(x_32, 1, x_31); -return x_32; -} -} -else -{ -lean_object* x_33; lean_object* x_34; lean_dec(x_3); -x_33 = lean_box(0); -x_34 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___lambda__1(x_2, x_9, x_19, x_33, x_4, x_5, x_6, x_7, x_8); -return x_34; -} -} +lean_dec(x_2); +return x_8; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___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_Elab_Inductive_0__Lean_Elab_Command_eqvFirstTypeResult___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; lean_object* x_8; -x_7 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_7, 0, x_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); -return x_8; +lean_object* x_9; +x_9 = l_Lean_Meta_isExprDefEq(x_3, x_1, x_4, x_5, x_6, x_7, x_8); +return x_9; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___closed__1() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_eqvFirstTypeResult(lean_object* x_1, 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_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___lambda__3___boxed), 6, 0); -return x_1; +lean_object* x_8; uint8_t x_9; lean_object* x_10; +x_8 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_eqvFirstTypeResult___lambda__1___boxed), 8, 1); +lean_closure_set(x_8, 0, x_2); +x_9 = 0; +x_10 = l_Lean_Meta_forallTelescopeReducing___at_Lean_Meta_getParamNames___spec__2___rarg(x_1, x_8, x_9, x_3, x_4, x_5, x_6, x_7); +return x_10; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs(lean_object* x_1, lean_object* x_2, lean_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_Inductive_0__Lean_Elab_Command_eqvFirstTypeResult___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_9; lean_object* x_10; uint8_t x_11; lean_object* x_12; -x_9 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___lambda__2___boxed), 8, 2); -lean_closure_set(x_9, 0, x_1); -lean_closure_set(x_9, 1, x_2); -x_10 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___closed__1; -x_11 = 0; -x_12 = l_Lean_Meta_transform___at_Lean_Meta_zetaReduce___spec__1(x_3, x_9, x_10, x_11, x_11, x_4, x_5, x_6, x_7, x_8); -return x_12; +lean_object* x_9; +x_9 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_eqvFirstTypeResult___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_2); +return x_9; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___spec__1___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_10; -x_10 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_1); -return x_10; +lean_object* x_11; +x_11 = lean_apply_9(x_1, x_4, x_5, x_2, x_3, x_6, x_7, x_8, x_9, x_10); +return x_11; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___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_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___spec__1___rarg(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_13; -x_13 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_2); -lean_dec(x_1); -return x_13; -} +lean_object* x_11; lean_object* x_12; +x_11 = lean_alloc_closure((void*)(l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___spec__1___rarg___lambda__1), 10, 3); +lean_closure_set(x_11, 0, x_2); +lean_closure_set(x_11, 1, x_4); +lean_closure_set(x_11, 2, x_5); +x_12 = l___private_Lean_Meta_Basic_0__Lean_Meta_forallTelescopeReducingImp___rarg(x_1, x_11, x_3, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_12) == 0) +{ +uint8_t x_13; +x_13 = !lean_is_exclusive(x_12); +if (x_13 == 0) +{ +return x_12; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +else { -lean_object* x_10; -x_10 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___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_1); -return x_10; +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_12, 0); +x_15 = lean_ctor_get(x_12, 1); +lean_inc(x_15); +lean_inc(x_14); +lean_dec(x_12); +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_14); +lean_ctor_set(x_16, 1, x_15); +return x_16; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___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: +else { -lean_object* x_9; -x_9 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_2); -lean_dec(x_1); -return x_9; -} +uint8_t x_17; +x_17 = !lean_is_exclusive(x_12); +if (x_17 == 0) +{ +return x_12; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___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: +else { -lean_object* x_7; -x_7 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___lambda__3(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_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_12, 0); +x_19 = lean_ctor_get(x_12, 1); +lean_inc(x_19); +lean_inc(x_18); +lean_dec(x_12); +x_20 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_20, 0, x_18); +lean_ctor_set(x_20, 1, x_19); +return x_20; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -lean_object* x_12; lean_object* x_13; -x_12 = l_Lean_mkAppN(x_1, x_2); -x_13 = lean_apply_8(x_3, x_12, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -return x_13; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__2___closed__1() { +LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___spec__1(lean_object* x_1) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("unexpected constructor resulting type, type expected", 52, 52); -return x_1; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___spec__1___rarg___boxed), 10, 0); +return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__2___closed__2() { +LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeCompatible___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___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_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__2___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +lean_object* x_12; +x_12 = lean_apply_10(x_1, x_4, x_5, x_6, x_2, x_3, x_7, x_8, x_9, x_10, x_11); +return x_12; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeCompatible___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___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_10; -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_1); -x_10 = l_Lean_Meta_isType(x_1, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_10) == 0) -{ -lean_object* x_11; uint8_t x_12; -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -x_12 = lean_unbox(x_11); -lean_dec(x_11); -if (x_12 == 0) -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_13 = lean_ctor_get(x_10, 1); -lean_inc(x_13); -lean_dec(x_10); -x_14 = l_Lean_indentExpr(x_1); -x_15 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__2___closed__2; -x_16 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_16, 0, x_15); -lean_ctor_set(x_16, 1, x_14); -x_17 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5; -x_18 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_18, 0, x_16); -lean_ctor_set(x_18, 1, x_17); -x_19 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_18, x_3, x_4, x_5, x_6, x_7, x_8, x_13); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -return x_19; -} -else +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_alloc_closure((void*)(l_Lean_Meta_forallTelescopeCompatible___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___spec__2___lambda__1), 11, 3); +lean_closure_set(x_12, 0, x_4); +lean_closure_set(x_12, 1, x_5); +lean_closure_set(x_12, 2, x_6); +x_13 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__8___closed__1; +x_14 = l_Lean_Meta_forallTelescopeCompatibleAux___rarg(x_12, x_3, x_1, x_2, x_13, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_14) == 0) { -uint8_t x_20; -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_20 = !lean_is_exclusive(x_10); -if (x_20 == 0) +uint8_t x_15; +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 0) { -lean_object* x_21; lean_object* x_22; -x_21 = lean_ctor_get(x_10, 0); -lean_dec(x_21); -x_22 = lean_box(0); -lean_ctor_set(x_10, 0, x_22); -return x_10; +return x_14; } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_10, 1); -lean_inc(x_23); -lean_dec(x_10); -x_24 = lean_box(0); -x_25 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_25, 0, x_24); -lean_ctor_set(x_25, 1, x_23); -return x_25; -} +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_14, 0); +x_17 = lean_ctor_get(x_14, 1); +lean_inc(x_17); +lean_inc(x_16); +lean_dec(x_14); +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_16); +lean_ctor_set(x_18, 1, x_17); +return x_18; } } else { -uint8_t x_26; -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_26 = !lean_is_exclusive(x_10); -if (x_26 == 0) +uint8_t x_19; +x_19 = !lean_is_exclusive(x_14); +if (x_19 == 0) { -return x_10; +return x_14; } else { -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_10, 0); -x_28 = lean_ctor_get(x_10, 1); -lean_inc(x_28); -lean_inc(x_27); -lean_dec(x_10); -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_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; } } } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__3___closed__1() { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__1___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("unexpected constructor resulting type", 37, 37); +x_1 = lean_mk_string_unchecked("resulting universe mismatch, given", 34, 34); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__3___closed__2() { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__3___closed__1; +x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__1___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___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) { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__1___closed__3() { _start: { -lean_object* x_11; uint8_t x_12; -x_11 = l_Lean_Expr_getAppFn(x_3); -x_12 = lean_expr_eqv(x_11, x_1); -lean_dec(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; -x_13 = l_Lean_indentExpr(x_3); -x_14 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__3___closed__2; -x_15 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_15, 0, x_14); -lean_ctor_set(x_15, 1, x_13); -x_16 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5; -x_17 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_17, 0, x_15); -lean_ctor_set(x_17, 1, x_16); -x_18 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_17, 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); -x_19 = !lean_is_exclusive(x_18); -if (x_19 == 0) -{ -return x_18; -} -else -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_18, 0); -x_21 = lean_ctor_get(x_18, 1); -lean_inc(x_21); -lean_inc(x_20); -lean_dec(x_18); -x_22 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_22, 0, x_20); -lean_ctor_set(x_22, 1, x_21); -return x_22; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("\nexpected type", 14, 14); +return x_1; } } -else +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__1___closed__4() { +_start: { -lean_object* x_23; lean_object* x_24; -x_23 = lean_box(0); -x_24 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__2(x_3, x_23, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_24; -} +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__1___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___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_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___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_14; uint8_t x_15; lean_object* x_16; -x_14 = 0; -x_15 = 0; -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); +lean_object* x_11; lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -x_16 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_14, x_15, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_16) == 0) +lean_inc(x_6); +x_11 = l_Lean_Meta_whnfD(x_1, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_11) == 0) { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_17 = lean_ctor_get(x_16, 1); -lean_inc(x_17); -lean_dec(x_16); -x_18 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_1, x_7, x_8, x_9, x_10, x_11, x_12, 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); +lean_object* x_12; +x_12 = lean_ctor_get(x_11, 0); lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -x_21 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs(x_2, x_3, x_19, x_9, x_10, x_11, x_12, x_20); -if (lean_obj_tag(x_21) == 0) +if (lean_obj_tag(x_12) == 3) { -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_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__3___boxed), 10, 1); -lean_closure_set(x_24, 0, x_4); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); +lean_object* x_13; lean_object* x_14; +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_22); -x_25 = l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___spec__1___rarg(x_22, x_24, x_15, x_7, x_8, x_9, x_10, x_11, x_12, x_23); -if (lean_obj_tag(x_25) == 0) +lean_inc(x_6); +lean_inc(x_12); +lean_inc(x_3); +x_14 = l_Lean_Meta_isExprDefEq(x_3, x_12, x_6, x_7, x_8, x_9, x_13); +if (lean_obj_tag(x_14) == 0) { -lean_object* x_26; lean_object* x_27; -x_26 = lean_ctor_get(x_25, 1); -lean_inc(x_26); -lean_dec(x_25); -x_27 = lean_apply_8(x_5, x_22, x_7, x_8, x_9, x_10, x_11, x_12, x_26); +lean_object* x_15; uint8_t x_16; +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_unbox(x_15); +lean_dec(x_15); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_17 = lean_ctor_get(x_14, 1); +lean_inc(x_17); +lean_dec(x_14); +x_18 = l_Lean_indentExpr(x_12); +x_19 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__1___closed__2; +x_20 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_20, 0, x_19); +lean_ctor_set(x_20, 1, x_18); +x_21 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__1___closed__4; +x_22 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_22, 0, x_20); +lean_ctor_set(x_22, 1, x_21); +x_23 = l_Lean_indentExpr(x_3); +x_24 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); +x_25 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +x_26 = lean_alloc_ctor(7, 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_Term_throwErrorIfErrors___spec__1(x_26, x_4, x_5, x_6, x_7, x_8, x_9, x_17); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); return x_27; } else { uint8_t x_28; -lean_dec(x_22); 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); -x_28 = !lean_is_exclusive(x_25); +lean_dec(x_6); +lean_dec(x_4); +lean_dec(x_3); +x_28 = !lean_is_exclusive(x_14); if (x_28 == 0) { -return x_25; +lean_object* x_29; lean_object* x_30; +x_29 = lean_ctor_get(x_14, 0); +lean_dec(x_29); +x_30 = lean_box(0); +lean_ctor_set(x_14, 0, x_30); +return x_14; } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_25, 0); -x_30 = lean_ctor_get(x_25, 1); -lean_inc(x_30); -lean_inc(x_29); -lean_dec(x_25); -x_31 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_31, 0, x_29); -lean_ctor_set(x_31, 1, x_30); -return x_31; +lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_31 = lean_ctor_get(x_14, 1); +lean_inc(x_31); +lean_dec(x_14); +x_32 = lean_box(0); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_31); +return x_33; } } } else { -uint8_t x_32; +uint8_t x_34; 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_6); lean_dec(x_4); -x_32 = !lean_is_exclusive(x_21); -if (x_32 == 0) +lean_dec(x_3); +x_34 = !lean_is_exclusive(x_14); +if (x_34 == 0) { -return x_21; +return x_14; } else { -lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_33 = lean_ctor_get(x_21, 0); -x_34 = lean_ctor_get(x_21, 1); -lean_inc(x_34); -lean_inc(x_33); -lean_dec(x_21); -x_35 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_35, 0, x_33); -lean_ctor_set(x_35, 1, x_34); -return x_35; +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_14, 0); +x_36 = lean_ctor_get(x_14, 1); +lean_inc(x_36); +lean_inc(x_35); +lean_dec(x_14); +x_37 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +return x_37; } } } else { -uint8_t x_36; +lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_dec(x_12); +lean_dec(x_3); +x_38 = lean_ctor_get(x_11, 1); +lean_inc(x_38); lean_dec(x_11); -lean_dec(x_10); +x_39 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___rarg___closed__2; +x_40 = l_Lean_throwError___at_Lean_Elab_Term_throwErrorIfErrors___spec__1(x_39, x_4, x_5, x_6, x_7, x_8, x_9, x_38); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_5); +lean_dec(x_6); +return x_40; +} +} +else +{ +uint8_t x_41; +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_36 = !lean_is_exclusive(x_16); -if (x_36 == 0) +x_41 = !lean_is_exclusive(x_11); +if (x_41 == 0) { -return x_16; +return x_11; } else { -lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_37 = lean_ctor_get(x_16, 0); -x_38 = lean_ctor_get(x_16, 1); -lean_inc(x_38); -lean_inc(x_37); -lean_dec(x_16); -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_11, 0); +x_43 = lean_ctor_get(x_11, 1); +lean_inc(x_43); +lean_inc(x_42); +lean_dec(x_11); +x_44 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_44, 0, x_42); +lean_ctor_set(x_44, 1, x_43); +return x_44; } } } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__1() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___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_1; -x_1 = lean_mk_string_unchecked("constructor resulting type must be specified in inductive family declaration", 76, 76); -return x_1; +lean_object* x_11; uint8_t x_12; lean_object* x_13; +x_11 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__1___boxed), 10, 1); +lean_closure_set(x_11, 0, x_3); +x_12 = 0; +x_13 = l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___spec__1___rarg(x_1, x_11, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_13; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__2() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +lean_object* x_11; uint8_t x_12; lean_object* x_13; +x_11 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__2___boxed), 10, 1); +lean_closure_set(x_11, 0, x_3); +x_12 = 0; +x_13 = l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___spec__1___rarg(x_2, x_11, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_13; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__3() { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("elabType ", 9, 9); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__3___boxed), 10, 0); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__3; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__5() { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___closed__2() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked(" : ", 3, 3); +x_1 = lean_mk_string_unchecked("invalid mutually inductive types, ", 34, 34); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__6() { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__5; +x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___closed__2; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__7() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked(" ", 1, 1); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__8() { -_start: +lean_object* x_11; lean_object* x_12; +x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___closed__1; +x_12 = l_Lean_Meta_forallTelescopeCompatible___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___spec__2(x_1, x_2, x_3, 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_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__7; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} +return x_12; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { -_start: +else { -lean_object* x_14; -x_14 = lean_ctor_get(x_5, 4); -lean_inc(x_14); -if (lean_obj_tag(x_14) == 0) +uint8_t x_13; +x_13 = !lean_is_exclusive(x_12); +if (x_13 == 0) { -lean_dec(x_5); -lean_dec(x_1); -if (x_4 == 0) +lean_object* x_14; uint8_t x_15; +x_14 = lean_ctor_get(x_12, 0); +x_15 = l_Lean_Exception_isInterrupt(x_14); +if (x_15 == 0) { -lean_object* x_15; lean_object* x_16; -x_15 = lean_box(0); -x_16 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__1(x_2, x_3, x_6, x_15, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_3); -return x_16; -} -else +uint8_t x_16; +x_16 = l_Lean_Exception_isRuntime(x_14); +if (x_16 == 0) { -lean_object* x_17; lean_object* x_18; uint8_t x_19; -lean_dec(x_6); -lean_dec(x_3); -lean_dec(x_2); -x_17 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__2; -x_18 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_17, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -x_19 = !lean_is_exclusive(x_18); -if (x_19 == 0) +if (lean_obj_tag(x_14) == 0) { -return x_18; -} -else +uint8_t x_17; +x_17 = !lean_is_exclusive(x_14); +if (x_17 == 0) { -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_18, 0); -x_21 = lean_ctor_get(x_18, 1); -lean_inc(x_21); -lean_inc(x_20); -lean_dec(x_18); -x_22 = lean_alloc_ctor(1, 2, 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); +x_19 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___closed__3; +x_20 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_20, 0, x_19); +lean_ctor_set(x_20, 1, x_18); +x_21 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +x_22 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_22, 0, x_20); lean_ctor_set(x_22, 1, x_21); -return x_22; -} -} +lean_ctor_set(x_14, 1, x_22); +return x_12; } else { -lean_object* x_23; lean_object* x_24; +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_23 = lean_ctor_get(x_14, 0); +x_24 = lean_ctor_get(x_14, 1); +lean_inc(x_24); lean_inc(x_23); lean_dec(x_14); -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_24 = l_Lean_Elab_Term_elabType(x_23, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_24) == 0) -{ -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; -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_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__3; -x_28 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_27, x_7, x_8, x_9, x_10, x_11, x_12, x_26); -x_29 = lean_ctor_get(x_28, 0); -lean_inc(x_29); -x_30 = lean_unbox(x_29); -lean_dec(x_29); -if (x_30 == 0) +x_25 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___closed__3; +x_26 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_24); +x_27 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +x_28 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +x_29 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_29, 0, x_23); +lean_ctor_set(x_29, 1, x_28); +lean_ctor_set(x_12, 0, x_29); +return x_12; +} +} +else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; -lean_dec(x_5); -x_31 = lean_ctor_get(x_28, 1); -lean_inc(x_31); -lean_dec(x_28); -x_32 = lean_box(0); -x_33 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__4(x_25, x_1, x_3, x_2, x_6, x_32, x_7, x_8, x_9, x_10, x_11, x_12, x_31); -return x_33; +return x_12; +} } else { -uint8_t x_34; -x_34 = !lean_is_exclusive(x_28); -if (x_34 == 0) +return x_12; +} +} +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; -x_35 = lean_ctor_get(x_28, 1); -x_36 = lean_ctor_get(x_28, 0); -lean_dec(x_36); -x_37 = lean_ctor_get(x_5, 2); -lean_inc(x_37); -lean_dec(x_5); -x_38 = l_Lean_MessageData_ofName(x_37); -x_39 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__4; -lean_ctor_set_tag(x_28, 7); -lean_ctor_set(x_28, 1, x_38); -lean_ctor_set(x_28, 0, x_39); -x_40 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__6; -x_41 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_41, 0, x_28); -lean_ctor_set(x_41, 1, x_40); -lean_inc(x_25); -x_42 = l_Lean_MessageData_ofExpr(x_25); -x_43 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_43, 0, x_41); -lean_ctor_set(x_43, 1, x_42); -x_44 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__8; -x_45 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_45, 0, x_43); -lean_ctor_set(x_45, 1, x_44); -x_46 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_27, x_45, x_7, x_8, x_9, x_10, x_11, x_12, x_35); -x_47 = lean_ctor_get(x_46, 0); -lean_inc(x_47); -x_48 = lean_ctor_get(x_46, 1); -lean_inc(x_48); -lean_dec(x_46); -x_49 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__4(x_25, x_1, x_3, x_2, x_6, x_47, x_7, x_8, x_9, x_10, x_11, x_12, x_48); -lean_dec(x_47); -return x_49; +return x_12; +} } else { -lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; -x_50 = lean_ctor_get(x_28, 1); -lean_inc(x_50); -lean_dec(x_28); -x_51 = lean_ctor_get(x_5, 2); -lean_inc(x_51); -lean_dec(x_5); -x_52 = l_Lean_MessageData_ofName(x_51); -x_53 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__4; -x_54 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_54, 0, x_53); -lean_ctor_set(x_54, 1, x_52); -x_55 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__6; -x_56 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_56, 0, x_54); -lean_ctor_set(x_56, 1, x_55); -lean_inc(x_25); -x_57 = l_Lean_MessageData_ofExpr(x_25); -x_58 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_58, 0, x_56); -lean_ctor_set(x_58, 1, x_57); -x_59 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__8; -x_60 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_60, 0, x_58); -lean_ctor_set(x_60, 1, x_59); -x_61 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_27, x_60, x_7, x_8, x_9, x_10, x_11, x_12, x_50); -x_62 = lean_ctor_get(x_61, 0); -lean_inc(x_62); -x_63 = lean_ctor_get(x_61, 1); -lean_inc(x_63); -lean_dec(x_61); -x_64 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__4(x_25, x_1, x_3, x_2, x_6, x_62, x_7, x_8, x_9, x_10, x_11, x_12, x_63); -lean_dec(x_62); -return x_64; +lean_object* x_30; lean_object* x_31; uint8_t x_32; +x_30 = lean_ctor_get(x_12, 0); +x_31 = lean_ctor_get(x_12, 1); +lean_inc(x_31); +lean_inc(x_30); +lean_dec(x_12); +x_32 = l_Lean_Exception_isInterrupt(x_30); +if (x_32 == 0) +{ +uint8_t x_33; +x_33 = l_Lean_Exception_isRuntime(x_30); +if (x_33 == 0) +{ +if (lean_obj_tag(x_30) == 0) +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_34 = lean_ctor_get(x_30, 0); +lean_inc(x_34); +x_35 = lean_ctor_get(x_30, 1); +lean_inc(x_35); +if (lean_is_exclusive(x_30)) { + lean_ctor_release(x_30, 0); + lean_ctor_release(x_30, 1); + x_36 = x_30; +} else { + lean_dec_ref(x_30); + x_36 = lean_box(0); } +x_37 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___closed__3; +x_38 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_38, 0, x_37); +lean_ctor_set(x_38, 1, x_35); +x_39 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +x_40 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +if (lean_is_scalar(x_36)) { + x_41 = lean_alloc_ctor(0, 2, 0); +} else { + x_41 = x_36; } +lean_ctor_set(x_41, 0, x_34); +lean_ctor_set(x_41, 1, x_40); +x_42 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_42, 0, x_41); +lean_ctor_set(x_42, 1, x_31); +return x_42; } else { -uint8_t x_65; -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_65 = !lean_is_exclusive(x_24); -if (x_65 == 0) +lean_object* x_43; +x_43 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_43, 0, x_30); +lean_ctor_set(x_43, 1, x_31); +return x_43; +} +} +else { -return x_24; +lean_object* x_44; +x_44 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_44, 0, x_30); +lean_ctor_set(x_44, 1, x_31); +return x_44; +} } else { -lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_66 = lean_ctor_get(x_24, 0); -x_67 = lean_ctor_get(x_24, 1); -lean_inc(x_67); -lean_inc(x_66); -lean_dec(x_24); -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_45; +x_45 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_45, 0, x_30); +lean_ctor_set(x_45, 1, x_31); +return x_45; } } } } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_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_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___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) { +_start: +{ +uint8_t x_11; lean_object* x_12; +x_11 = lean_unbox(x_3); +lean_dec(x_3); +x_12 = l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___spec__1___rarg(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_Meta_forallTelescopeCompatible___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___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_2); +x_12 = l_Lean_Meta_forallTelescopeCompatible___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___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_3); return x_12; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_10; -x_10 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_4); +lean_object* x_11; +x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___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_2); -return x_10; +return x_11; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___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_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; -x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_5); +x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___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_2); -lean_dec(x_1); return x_11; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___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_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_14; -x_14 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_6); -return x_14; +lean_object* x_11; +x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___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_1); +return x_11; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_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_14; lean_object* x_15; -x_14 = lean_unbox(x_4); -lean_dec(x_4); -x_15 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType(x_1, x_2, x_3, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -return x_15; +lean_object* x_11; +x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType(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 uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__1(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkHeader(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_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_5; -x_5 = lean_usize_dec_eq(x_3, x_4); -if (x_5 == 0) +lean_object* x_11; +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_1); +x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkTypeFor(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_11) == 0) { -lean_object* x_6; uint8_t x_7; -x_6 = lean_array_uget(x_2, x_3); -x_7 = l_Lean_Expr_isMVar(x_6); -if (x_7 == 0) +if (lean_obj_tag(x_3) == 0) { -size_t x_8; size_t x_9; +uint8_t x_12; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); -x_8 = 1; -x_9 = lean_usize_add(x_3, x_8); -x_3 = x_9; -goto _start; +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_1); +x_12 = !lean_is_exclusive(x_11); +if (x_12 == 0) +{ +return x_11; } else { -lean_object* x_11; uint8_t x_12; -x_11 = l_Lean_Expr_mvarId_x21(x_6); -lean_dec(x_6); -x_12 = lean_name_eq(x_11, x_1); -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; +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 = 1; -return x_16; -} -} +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_16 = lean_ctor_get(x_11, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_11, 1); +lean_inc(x_17); +lean_dec(x_11); +x_18 = lean_ctor_get(x_3, 0); +lean_inc(x_18); +lean_dec(x_3); +x_19 = lean_ctor_get(x_1, 0); +lean_inc(x_19); +lean_dec(x_1); +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +lean_dec(x_19); +x_21 = !lean_is_exclusive(x_8); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_8, 5); +x_23 = l_Lean_replaceRef(x_20, x_22); +lean_dec(x_22); +lean_dec(x_20); +lean_ctor_set(x_8, 5, x_23); +lean_inc(x_18); +x_24 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType(x_16, x_18, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_17); +if (lean_obj_tag(x_24) == 0) +{ +uint8_t x_25; +x_25 = !lean_is_exclusive(x_24); +if (x_25 == 0) +{ +lean_object* x_26; +x_26 = lean_ctor_get(x_24, 0); +lean_dec(x_26); +lean_ctor_set(x_24, 0, x_18); +return x_24; } else { -uint8_t x_17; -x_17 = 0; -return x_17; -} +lean_object* x_27; lean_object* x_28; +x_27 = lean_ctor_get(x_24, 1); +lean_inc(x_27); +lean_dec(x_24); +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_18); +lean_ctor_set(x_28, 1, x_27); +return x_28; } } -LEAN_EXPORT uint8_t l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__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_29; +lean_dec(x_18); +x_29 = !lean_is_exclusive(x_24); +if (x_29 == 0) { -uint8_t x_6; -lean_dec(x_3); -x_6 = 0; -return x_6; +return x_24; } else { -size_t x_7; size_t x_8; uint8_t x_9; -x_7 = 0; -x_8 = lean_usize_of_nat(x_3); -lean_dec(x_3); -x_9 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__1(x_2, x_1, x_7, x_8); -return x_9; +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_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: +else { -lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_11 = lean_ctor_get(x_1, 2); -lean_inc(x_11); -x_12 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_12, 0, x_11); -lean_ctor_set(x_12, 1, x_2); -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_12); -lean_ctor_set(x_13, 1, x_10); -return x_13; +lean_object* x_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_45; uint8_t x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_33 = lean_ctor_get(x_8, 0); +x_34 = lean_ctor_get(x_8, 1); +x_35 = lean_ctor_get(x_8, 2); +x_36 = lean_ctor_get(x_8, 3); +x_37 = lean_ctor_get(x_8, 4); +x_38 = lean_ctor_get(x_8, 5); +x_39 = lean_ctor_get(x_8, 6); +x_40 = lean_ctor_get(x_8, 7); +x_41 = lean_ctor_get(x_8, 8); +x_42 = lean_ctor_get(x_8, 9); +x_43 = lean_ctor_get(x_8, 10); +x_44 = lean_ctor_get_uint8(x_8, sizeof(void*)*12); +x_45 = lean_ctor_get(x_8, 11); +x_46 = lean_ctor_get_uint8(x_8, sizeof(void*)*12 + 1); +lean_inc(x_45); +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_dec(x_8); +x_47 = l_Lean_replaceRef(x_20, x_38); +lean_dec(x_38); +lean_dec(x_20); +x_48 = lean_alloc_ctor(0, 12, 2); +lean_ctor_set(x_48, 0, x_33); +lean_ctor_set(x_48, 1, x_34); +lean_ctor_set(x_48, 2, x_35); +lean_ctor_set(x_48, 3, x_36); +lean_ctor_set(x_48, 4, x_37); +lean_ctor_set(x_48, 5, x_47); +lean_ctor_set(x_48, 6, x_39); +lean_ctor_set(x_48, 7, x_40); +lean_ctor_set(x_48, 8, x_41); +lean_ctor_set(x_48, 9, x_42); +lean_ctor_set(x_48, 10, x_43); +lean_ctor_set(x_48, 11, x_45); +lean_ctor_set_uint8(x_48, sizeof(void*)*12, x_44); +lean_ctor_set_uint8(x_48, sizeof(void*)*12 + 1, x_46); +lean_inc(x_18); +x_49 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType(x_16, x_18, x_2, x_4, x_5, x_6, x_7, x_48, x_9, x_17); +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, 1); +lean_inc(x_50); +if (lean_is_exclusive(x_49)) { + lean_ctor_release(x_49, 0); + lean_ctor_release(x_49, 1); + x_51 = x_49; +} else { + lean_dec_ref(x_49); + x_51 = lean_box(0); } +if (lean_is_scalar(x_51)) { + x_52 = lean_alloc_ctor(0, 2, 0); +} else { + x_52 = x_51; } -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { -_start: -{ -lean_object* x_15; uint8_t x_16; uint8_t x_17; uint8_t x_18; lean_object* x_19; -x_15 = l_Array_append___rarg(x_1, x_2); -x_16 = 0; -x_17 = 1; -x_18 = 1; -x_19 = l_Lean_Meta_mkForallFVars(x_15, x_3, x_16, x_17, x_18, x_10, x_11, x_12, x_13, x_14); -if (lean_obj_tag(x_19) == 0) -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_19, 1); -lean_inc(x_21); -lean_dec(x_19); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -x_22 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs(x_20, x_10, x_11, x_12, x_13, x_21); -if (lean_obj_tag(x_22) == 0) -{ -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -x_24 = lean_ctor_get(x_22, 1); -lean_inc(x_24); -lean_dec(x_22); -x_25 = l_Lean_Meta_mkForallFVars(x_4, x_23, x_16, x_17, x_18, x_10, x_11, x_12, x_13, x_24); -if (lean_obj_tag(x_25) == 0) -{ -lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; -x_26 = lean_ctor_get(x_25, 0); -lean_inc(x_26); -x_27 = lean_ctor_get(x_25, 1); -lean_inc(x_27); -lean_dec(x_25); -lean_inc(x_5); -x_28 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_5, x_8, x_9, x_10, x_11, x_12, x_13, x_27); -x_29 = lean_ctor_get(x_28, 0); -lean_inc(x_29); -x_30 = lean_unbox(x_29); -lean_dec(x_29); -if (x_30 == 0) -{ -lean_object* x_31; lean_object* x_32; lean_object* x_33; -lean_dec(x_5); -x_31 = lean_ctor_get(x_28, 1); -lean_inc(x_31); -lean_dec(x_28); -x_32 = lean_box(0); -x_33 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__2(x_6, x_26, x_32, x_8, x_9, x_10, x_11, x_12, x_13, x_31); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_6); -return x_33; +lean_ctor_set(x_52, 0, x_18); +lean_ctor_set(x_52, 1, x_50); +return x_52; } else { -uint8_t x_34; -x_34 = !lean_is_exclusive(x_28); -if (x_34 == 0) -{ -lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; -x_35 = lean_ctor_get(x_28, 1); -x_36 = lean_ctor_get(x_28, 0); -lean_dec(x_36); -x_37 = lean_ctor_get(x_6, 2); -lean_inc(x_37); -x_38 = l_Lean_MessageData_ofName(x_37); -x_39 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5; -lean_ctor_set_tag(x_28, 7); -lean_ctor_set(x_28, 1, x_38); -lean_ctor_set(x_28, 0, x_39); -x_40 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__6; -x_41 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_41, 0, x_28); -lean_ctor_set(x_41, 1, x_40); -lean_inc(x_26); -x_42 = l_Lean_MessageData_ofExpr(x_26); -x_43 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_43, 0, x_41); -lean_ctor_set(x_43, 1, x_42); -x_44 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_44, 0, x_43); -lean_ctor_set(x_44, 1, x_39); -x_45 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_5, x_44, x_8, x_9, x_10, x_11, x_12, x_13, x_35); -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_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__2(x_6, x_26, x_46, x_8, x_9, x_10, x_11, x_12, x_13, x_47); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_46); -lean_dec(x_6); -return x_48; +lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; +lean_dec(x_18); +x_53 = lean_ctor_get(x_49, 0); +lean_inc(x_53); +x_54 = lean_ctor_get(x_49, 1); +lean_inc(x_54); +if (lean_is_exclusive(x_49)) { + lean_ctor_release(x_49, 0); + lean_ctor_release(x_49, 1); + x_55 = x_49; +} else { + lean_dec_ref(x_49); + x_55 = lean_box(0); +} +if (lean_is_scalar(x_55)) { + x_56 = lean_alloc_ctor(1, 2, 0); +} else { + x_56 = x_55; +} +lean_ctor_set(x_56, 0, x_53); +lean_ctor_set(x_56, 1, x_54); +return x_56; } -else -{ -lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_49 = lean_ctor_get(x_28, 1); -lean_inc(x_49); -lean_dec(x_28); -x_50 = lean_ctor_get(x_6, 2); -lean_inc(x_50); -x_51 = l_Lean_MessageData_ofName(x_50); -x_52 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5; -x_53 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_53, 0, x_52); -lean_ctor_set(x_53, 1, x_51); -x_54 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__6; -x_55 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_55, 0, x_53); -lean_ctor_set(x_55, 1, x_54); -lean_inc(x_26); -x_56 = l_Lean_MessageData_ofExpr(x_26); -x_57 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_57, 0, x_55); -lean_ctor_set(x_57, 1, x_56); -x_58 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_58, 0, x_57); -lean_ctor_set(x_58, 1, x_52); -x_59 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_5, x_58, x_8, x_9, x_10, x_11, x_12, x_13, x_49); -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_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__2(x_6, x_26, x_60, x_8, x_9, x_10, x_11, x_12, x_13, x_61); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_60); -lean_dec(x_6); -return x_62; } } } else { -uint8_t x_63; -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); +uint8_t x_57; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -x_63 = !lean_is_exclusive(x_25); -if (x_63 == 0) +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_57 = !lean_is_exclusive(x_11); +if (x_57 == 0) { -return x_25; +return x_11; } else { -lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_64 = lean_ctor_get(x_25, 0); -x_65 = lean_ctor_get(x_25, 1); -lean_inc(x_65); -lean_inc(x_64); -lean_dec(x_25); -x_66 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_66, 0, x_64); -lean_ctor_set(x_66, 1, x_65); -return x_66; +lean_object* x_58; lean_object* x_59; lean_object* x_60; +x_58 = lean_ctor_get(x_11, 0); +x_59 = lean_ctor_get(x_11, 1); +lean_inc(x_59); +lean_inc(x_58); +lean_dec(x_11); +x_60 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_60, 0, x_58); +lean_ctor_set(x_60, 1, x_59); +return x_60; } } } -else +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkHeader___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_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_67; -lean_dec(x_13); +lean_object* x_11; +x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkHeader(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_2); +return x_11; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkHeaders(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; uint8_t x_13; +x_12 = lean_array_get_size(x_1); +x_13 = lean_nat_dec_lt(x_3, x_12); lean_dec(x_12); -lean_dec(x_11); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_67 = !lean_is_exclusive(x_22); -if (x_67 == 0) -{ -return x_22; +lean_dec(x_3); +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_11); +return x_15; } else { -lean_object* x_68; lean_object* x_69; lean_object* x_70; -x_68 = lean_ctor_get(x_22, 0); -x_69 = lean_ctor_get(x_22, 1); -lean_inc(x_69); -lean_inc(x_68); -lean_dec(x_22); -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_16; lean_object* x_17; +x_16 = lean_array_fget(x_1, 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_5); +x_17 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkHeader(x_16, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_17) == 0) +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); +lean_dec(x_17); +x_20 = lean_unsigned_to_nat(1u); +x_21 = lean_nat_add(x_3, x_20); +lean_dec(x_3); +x_22 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_22, 0, x_18); +x_3 = x_21; +x_4 = x_22; +x_11 = x_19; +goto _start; } else { -uint8_t x_71; -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); +uint8_t x_24; lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); -x_71 = !lean_is_exclusive(x_19); -if (x_71 == 0) +lean_dec(x_3); +x_24 = !lean_is_exclusive(x_17); +if (x_24 == 0) { -return x_19; +return x_17; } else { -lean_object* x_72; lean_object* x_73; lean_object* x_74; -x_72 = lean_ctor_get(x_19, 0); -x_73 = lean_ctor_get(x_19, 1); -lean_inc(x_73); -lean_inc(x_72); -lean_dec(x_19); -x_74 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_74, 0, x_72); -lean_ctor_set(x_74, 1, x_73); -return x_74; +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_17, 0); +x_26 = lean_ctor_get(x_17, 1); +lean_inc(x_26); +lean_inc(x_25); +lean_dec(x_17); +x_27 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +return x_27; } } } } -static lean_object* _init_l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__4___closed__1() { +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkHeaders___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("extraCtorParams: ", 17, 17); -return x_1; +lean_object* x_12; +x_12 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkHeaders(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_2); +lean_dec(x_1); +return x_12; } } -static lean_object* _init_l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__4___closed__2() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeader___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__4___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +lean_object* x_10; +x_10 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_10, 0, x_1); +lean_ctor_set(x_10, 1, x_9); +return x_10; } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___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_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_Inductive_0__Lean_Elab_Command_elabHeader(lean_object* x_1, lean_object* x_2, lean_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_12; uint8_t x_13; lean_object* x_14; -x_12 = 1; -x_13 = 0; -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = lean_unsigned_to_nat(0u); +x_10 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__8___closed__1; lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_14 = l_Lean_Elab_Term_synthesizeSyntheticMVars(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_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux(x_1, x_9, x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_11) == 0) { -lean_object* x_15; lean_object* x_16; -x_15 = lean_ctor_get(x_14, 1); -lean_inc(x_15); -lean_dec(x_14); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_5); -x_16 = l_Lean_Elab_Term_addAutoBoundImplicits(x_1, x_5, x_6, x_7, x_8, x_9, x_10, x_15); -if (lean_obj_tag(x_16) == 0) +uint8_t x_12; +x_12 = !lean_is_exclusive(x_11); +if (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; lean_object* x_24; lean_object* x_25; uint8_t x_26; -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_16, 1); -lean_inc(x_18); -lean_dec(x_16); -lean_inc(x_17); -x_19 = lean_alloc_closure((void*)(l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__1___boxed), 2, 1); -lean_closure_set(x_19, 0, x_17); -lean_inc(x_4); -x_20 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_18); +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_11, 0); +x_14 = lean_ctor_get(x_11, 1); +x_15 = lean_array_get_size(x_13); +x_16 = lean_unsigned_to_nat(1u); +x_17 = lean_nat_dec_lt(x_16, x_15); +lean_dec(x_15); +if (x_17 == 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); +return x_11; +} +else +{ +lean_object* x_18; +lean_free_object(x_11); +lean_inc(x_6); +lean_inc(x_2); +x_18 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe(x_13, x_2, x_3, x_4, x_5, x_6, x_7, x_14); +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); +lean_inc(x_6); +lean_inc(x_2); +x_20 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams(x_13, x_2, x_3, x_4, x_5, x_6, x_7, x_19); +if (lean_obj_tag(x_20) == 0) +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; x_21 = lean_ctor_get(x_20, 0); lean_inc(x_21); x_22 = lean_ctor_get(x_20, 1); lean_inc(x_22); lean_dec(x_20); x_23 = lean_box(0); -x_24 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__3___closed__1; -x_25 = l_Lean_Elab_Term_collectUnassignedMVars(x_21, x_24, x_19, x_5, x_6, x_7, x_8, x_9, x_10, x_22); -x_26 = !lean_is_exclusive(x_25); -if (x_26 == 0) -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; -x_27 = lean_ctor_get(x_25, 0); -x_28 = lean_ctor_get(x_25, 1); -x_29 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__3; -x_30 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_29, x_5, x_6, x_7, x_8, x_9, x_10, x_28); -x_31 = lean_ctor_get(x_30, 0); -lean_inc(x_31); -x_32 = lean_unbox(x_31); -lean_dec(x_31); -if (x_32 == 0) -{ -lean_object* x_33; lean_object* x_34; lean_object* x_35; -lean_free_object(x_25); -x_33 = lean_ctor_get(x_30, 1); -lean_inc(x_33); -lean_dec(x_30); -x_34 = lean_box(0); -x_35 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__3(x_27, x_17, x_4, x_2, x_29, x_3, x_34, x_5, x_6, x_7, x_8, x_9, x_10, x_33); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_17); -return x_35; -} -else +x_24 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkHeaders(x_13, x_21, x_9, x_23, x_2, x_3, x_4, x_5, x_6, x_7, x_22); +lean_dec(x_21); +if (lean_obj_tag(x_24) == 0) { -uint8_t x_36; -x_36 = !lean_is_exclusive(x_30); -if (x_36 == 0) +uint8_t x_25; +x_25 = !lean_is_exclusive(x_24); +if (x_25 == 0) { -lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_37 = lean_ctor_get(x_30, 1); -x_38 = lean_ctor_get(x_30, 0); -lean_dec(x_38); -lean_inc(x_27); -x_39 = lean_array_to_list(x_27); -x_40 = l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(x_39, x_23); -x_41 = l_Lean_MessageData_ofList(x_40); -x_42 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__4___closed__2; -lean_ctor_set_tag(x_30, 7); -lean_ctor_set(x_30, 1, x_41); -lean_ctor_set(x_30, 0, x_42); -x_43 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5; -lean_ctor_set_tag(x_25, 7); -lean_ctor_set(x_25, 1, x_43); -lean_ctor_set(x_25, 0, x_30); -x_44 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_29, x_25, x_5, x_6, x_7, x_8, x_9, x_10, x_37); -x_45 = lean_ctor_get(x_44, 0); -lean_inc(x_45); -x_46 = lean_ctor_get(x_44, 1); -lean_inc(x_46); -lean_dec(x_44); -x_47 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__3(x_27, x_17, x_4, x_2, x_29, x_3, x_45, x_5, x_6, x_7, x_8, x_9, x_10, x_46); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_45); -lean_dec(x_17); -return x_47; +lean_object* x_26; +x_26 = lean_ctor_get(x_24, 0); +lean_dec(x_26); +lean_ctor_set(x_24, 0, x_13); +return x_24; } 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; -x_48 = lean_ctor_get(x_30, 1); -lean_inc(x_48); -lean_dec(x_30); +lean_object* x_27; lean_object* x_28; +x_27 = lean_ctor_get(x_24, 1); lean_inc(x_27); -x_49 = lean_array_to_list(x_27); -x_50 = l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(x_49, x_23); -x_51 = l_Lean_MessageData_ofList(x_50); -x_52 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__4___closed__2; -x_53 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_53, 0, x_52); -lean_ctor_set(x_53, 1, x_51); -x_54 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5; -lean_ctor_set_tag(x_25, 7); -lean_ctor_set(x_25, 1, x_54); -lean_ctor_set(x_25, 0, x_53); -x_55 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_29, x_25, x_5, x_6, x_7, x_8, x_9, x_10, x_48); -x_56 = lean_ctor_get(x_55, 0); -lean_inc(x_56); -x_57 = lean_ctor_get(x_55, 1); -lean_inc(x_57); -lean_dec(x_55); -x_58 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__3(x_27, x_17, x_4, x_2, x_29, x_3, x_56, x_5, x_6, x_7, x_8, x_9, x_10, x_57); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_56); -lean_dec(x_17); -return x_58; -} +lean_dec(x_24); +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_13); +lean_ctor_set(x_28, 1, x_27); +return x_28; } } else { -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_ctor_get(x_25, 0); -x_60 = lean_ctor_get(x_25, 1); -lean_inc(x_60); -lean_inc(x_59); -lean_dec(x_25); -x_61 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__3; -x_62 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_61, x_5, x_6, x_7, x_8, x_9, x_10, x_60); -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) +uint8_t x_29; +lean_dec(x_13); +x_29 = !lean_is_exclusive(x_24); +if (x_29 == 0) { -lean_object* x_65; lean_object* x_66; lean_object* x_67; -x_65 = lean_ctor_get(x_62, 1); -lean_inc(x_65); -lean_dec(x_62); -x_66 = lean_box(0); -x_67 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__3(x_59, x_17, x_4, x_2, x_61, x_3, x_66, x_5, x_6, x_7, x_8, x_9, x_10, x_65); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_17); -return x_67; +return x_24; } else { -lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; -x_68 = lean_ctor_get(x_62, 1); -lean_inc(x_68); -if (lean_is_exclusive(x_62)) { - lean_ctor_release(x_62, 0); - lean_ctor_release(x_62, 1); - x_69 = x_62; -} else { - lean_dec_ref(x_62); - x_69 = lean_box(0); -} -lean_inc(x_59); -x_70 = lean_array_to_list(x_59); -x_71 = l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(x_70, x_23); -x_72 = l_Lean_MessageData_ofList(x_71); -x_73 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__4___closed__2; -if (lean_is_scalar(x_69)) { - x_74 = lean_alloc_ctor(7, 2, 0); -} else { - x_74 = x_69; - lean_ctor_set_tag(x_74, 7); -} -lean_ctor_set(x_74, 0, x_73); -lean_ctor_set(x_74, 1, x_72); -x_75 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5; -x_76 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_76, 0, x_74); -lean_ctor_set(x_76, 1, x_75); -x_77 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_61, x_76, x_5, x_6, x_7, x_8, x_9, x_10, x_68); -x_78 = lean_ctor_get(x_77, 0); -lean_inc(x_78); -x_79 = lean_ctor_get(x_77, 1); -lean_inc(x_79); -lean_dec(x_77); -x_80 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__3(x_59, x_17, x_4, x_2, x_61, x_3, x_78, x_5, x_6, x_7, x_8, x_9, x_10, x_79); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_78); -lean_dec(x_17); -return x_80; +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; } } } else { -uint8_t x_81; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); +uint8_t x_33; +lean_dec(x_13); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_81 = !lean_is_exclusive(x_16); -if (x_81 == 0) +x_33 = !lean_is_exclusive(x_20); +if (x_33 == 0) { -return x_16; +return x_20; } else { -lean_object* x_82; lean_object* x_83; lean_object* x_84; -x_82 = lean_ctor_get(x_16, 0); -x_83 = lean_ctor_get(x_16, 1); -lean_inc(x_83); -lean_inc(x_82); -lean_dec(x_16); -x_84 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_84, 0, x_82); -lean_ctor_set(x_84, 1, x_83); -return x_84; +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_20, 0); +x_35 = lean_ctor_get(x_20, 1); +lean_inc(x_35); +lean_inc(x_34); +lean_dec(x_20); +x_36 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_36, 0, x_34); +lean_ctor_set(x_36, 1, x_35); +return x_36; } } } else { -uint8_t x_85; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); +uint8_t x_37; +lean_dec(x_13); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_85 = !lean_is_exclusive(x_14); -if (x_85 == 0) +x_37 = !lean_is_exclusive(x_18); +if (x_37 == 0) { -return x_14; +return x_18; } else { -lean_object* x_86; lean_object* x_87; lean_object* x_88; -x_86 = lean_ctor_get(x_14, 0); -x_87 = lean_ctor_get(x_14, 1); -lean_inc(x_87); -lean_inc(x_86); -lean_dec(x_14); -x_88 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_88, 0, x_86); -lean_ctor_set(x_88, 1, x_87); -return x_88; -} +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_18, 0); +x_39 = lean_ctor_get(x_18, 1); +lean_inc(x_39); +lean_inc(x_38); +lean_dec(x_18); +x_40 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +return x_40; } } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__5(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) { -_start: -{ -lean_object* x_14; lean_object* x_15; uint8_t x_16; -x_14 = lean_ctor_get(x_1, 0); -lean_inc(x_14); -lean_inc(x_1); -lean_inc(x_2); -x_15 = lean_alloc_closure((void*)(l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__4___boxed), 11, 3); -lean_closure_set(x_15, 0, x_6); -lean_closure_set(x_15, 1, x_2); -lean_closure_set(x_15, 2, x_1); -x_16 = !lean_is_exclusive(x_11); -if (x_16 == 0) -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_11, 5); -x_18 = l_Lean_replaceRef(x_14, x_17); -lean_dec(x_17); -lean_dec(x_14); -lean_ctor_set(x_11, 5, x_18); -x_19 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType(x_3, x_4, x_2, x_5, x_1, x_15, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -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; uint8_t x_31; lean_object* x_32; uint8_t x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_20 = lean_ctor_get(x_11, 0); -x_21 = lean_ctor_get(x_11, 1); -x_22 = lean_ctor_get(x_11, 2); -x_23 = lean_ctor_get(x_11, 3); -x_24 = lean_ctor_get(x_11, 4); -x_25 = lean_ctor_get(x_11, 5); -x_26 = lean_ctor_get(x_11, 6); -x_27 = lean_ctor_get(x_11, 7); -x_28 = lean_ctor_get(x_11, 8); -x_29 = lean_ctor_get(x_11, 9); -x_30 = lean_ctor_get(x_11, 10); -x_31 = lean_ctor_get_uint8(x_11, sizeof(void*)*12); -x_32 = lean_ctor_get(x_11, 11); -x_33 = lean_ctor_get_uint8(x_11, sizeof(void*)*12 + 1); -lean_inc(x_32); -lean_inc(x_30); -lean_inc(x_29); -lean_inc(x_28); -lean_inc(x_27); -lean_inc(x_26); -lean_inc(x_25); -lean_inc(x_24); -lean_inc(x_23); -lean_inc(x_22); -lean_inc(x_21); -lean_inc(x_20); +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_11, 0); +x_42 = lean_ctor_get(x_11, 1); +lean_inc(x_42); +lean_inc(x_41); lean_dec(x_11); -x_34 = l_Lean_replaceRef(x_14, x_25); -lean_dec(x_25); -lean_dec(x_14); -x_35 = lean_alloc_ctor(0, 12, 2); -lean_ctor_set(x_35, 0, x_20); -lean_ctor_set(x_35, 1, x_21); -lean_ctor_set(x_35, 2, x_22); -lean_ctor_set(x_35, 3, x_23); -lean_ctor_set(x_35, 4, x_24); -lean_ctor_set(x_35, 5, x_34); -lean_ctor_set(x_35, 6, x_26); -lean_ctor_set(x_35, 7, x_27); -lean_ctor_set(x_35, 8, x_28); -lean_ctor_set(x_35, 9, x_29); -lean_ctor_set(x_35, 10, x_30); -lean_ctor_set(x_35, 11, x_32); -lean_ctor_set_uint8(x_35, sizeof(void*)*12, x_31); -lean_ctor_set_uint8(x_35, sizeof(void*)*12 + 1, x_33); -x_36 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType(x_3, x_4, x_2, x_5, x_1, x_15, x_7, x_8, x_9, x_10, x_35, x_12, x_13); -return x_36; -} -} -} -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { -_start: -{ -if (lean_obj_tag(x_5) == 0) +x_43 = lean_array_get_size(x_41); +x_44 = lean_unsigned_to_nat(1u); +x_45 = lean_nat_dec_lt(x_44, x_43); +lean_dec(x_43); +if (x_45 == 0) { -lean_object* x_14; lean_object* x_15; -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); +lean_object* x_46; 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_14 = l_List_reverse___rarg(x_6); -x_15 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_15, 0, x_14); -lean_ctor_set(x_15, 1, x_13); -return x_15; +x_46 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_46, 0, x_41); +lean_ctor_set(x_46, 1, x_42); +return x_46; } else { -uint8_t x_16; -x_16 = !lean_is_exclusive(x_5); -if (x_16 == 0) +lean_object* x_47; +lean_inc(x_6); +lean_inc(x_2); +x_47 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe(x_41, x_2, x_3, x_4, x_5, x_6, x_7, x_42); +if (lean_obj_tag(x_47) == 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; -x_17 = lean_ctor_get(x_5, 0); -x_18 = lean_ctor_get(x_5, 1); -x_19 = lean_ctor_get(x_17, 3); -lean_inc(x_19); -x_20 = l_Lean_Syntax_getArgs(x_19); -lean_dec(x_19); -x_21 = lean_box(x_4); +lean_object* x_48; lean_object* x_49; +x_48 = lean_ctor_get(x_47, 1); +lean_inc(x_48); +lean_dec(x_47); +lean_inc(x_6); lean_inc(x_2); -lean_inc(x_1); -lean_inc(x_3); -x_22 = lean_alloc_closure((void*)(l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__5___boxed), 13, 5); -lean_closure_set(x_22, 0, x_17); -lean_closure_set(x_22, 1, x_3); -lean_closure_set(x_22, 2, x_1); -lean_closure_set(x_22, 3, x_2); -lean_closure_set(x_22, 4, x_21); -x_23 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabBinders___rarg), 9, 2); -lean_closure_set(x_23, 0, x_20); -lean_closure_set(x_23, 1, x_22); -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_24 = l_Lean_Elab_Term_withAutoBoundImplicit___rarg(x_23, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_24) == 0) +x_49 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams(x_41, x_2, x_3, x_4, x_5, x_6, x_7, x_48); +if (lean_obj_tag(x_49) == 0) { -lean_object* x_25; lean_object* x_26; -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_ctor_set(x_5, 1, x_6); -lean_ctor_set(x_5, 0, x_25); +lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; +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_box(0); +x_53 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkHeaders(x_41, x_50, x_9, x_52, x_2, x_3, x_4, x_5, x_6, x_7, x_51); +lean_dec(x_50); +if (lean_obj_tag(x_53) == 0) { -lean_object* _tmp_4 = x_18; -lean_object* _tmp_5 = x_5; -lean_object* _tmp_12 = x_26; -x_5 = _tmp_4; -x_6 = _tmp_5; -x_13 = _tmp_12; +lean_object* x_54; lean_object* x_55; lean_object* x_56; +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_53); + x_55 = lean_box(0); } -goto _start; +if (lean_is_scalar(x_55)) { + x_56 = lean_alloc_ctor(0, 2, 0); +} else { + x_56 = x_55; } -else -{ -uint8_t x_28; -lean_free_object(x_5); -lean_dec(x_18); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_28 = !lean_is_exclusive(x_24); -if (x_28 == 0) -{ -return x_24; +lean_ctor_set(x_56, 0, x_41); +lean_ctor_set(x_56, 1, x_54); +return x_56; } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_24, 0); -x_30 = lean_ctor_get(x_24, 1); -lean_inc(x_30); -lean_inc(x_29); -lean_dec(x_24); -x_31 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_31, 0, x_29); -lean_ctor_set(x_31, 1, x_30); -return x_31; +lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; +lean_dec(x_41); +x_57 = lean_ctor_get(x_53, 0); +lean_inc(x_57); +x_58 = lean_ctor_get(x_53, 1); +lean_inc(x_58); +if (lean_is_exclusive(x_53)) { + lean_ctor_release(x_53, 0); + lean_ctor_release(x_53, 1); + x_59 = x_53; +} else { + lean_dec_ref(x_53); + x_59 = lean_box(0); +} +if (lean_is_scalar(x_59)) { + x_60 = lean_alloc_ctor(1, 2, 0); +} else { + x_60 = x_59; } +lean_ctor_set(x_60, 0, x_57); +lean_ctor_set(x_60, 1, x_58); +return x_60; } } else { -lean_object* x_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_5, 0); -x_33 = lean_ctor_get(x_5, 1); -lean_inc(x_33); -lean_inc(x_32); +lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; +lean_dec(x_41); +lean_dec(x_7); +lean_dec(x_6); lean_dec(x_5); -x_34 = lean_ctor_get(x_32, 3); -lean_inc(x_34); -x_35 = l_Lean_Syntax_getArgs(x_34); -lean_dec(x_34); -x_36 = lean_box(x_4); -lean_inc(x_2); -lean_inc(x_1); -lean_inc(x_3); -x_37 = lean_alloc_closure((void*)(l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__5___boxed), 13, 5); -lean_closure_set(x_37, 0, x_32); -lean_closure_set(x_37, 1, x_3); -lean_closure_set(x_37, 2, x_1); -lean_closure_set(x_37, 3, x_2); -lean_closure_set(x_37, 4, x_36); -x_38 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabBinders___rarg), 9, 2); -lean_closure_set(x_38, 0, x_35); -lean_closure_set(x_38, 1, x_37); -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_39 = l_Lean_Elab_Term_withAutoBoundImplicit___rarg(x_38, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -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 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_42, 0, x_40); -lean_ctor_set(x_42, 1, x_6); -x_5 = x_33; -x_6 = x_42; -x_13 = x_41; -goto _start; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_61 = lean_ctor_get(x_49, 0); +lean_inc(x_61); +x_62 = lean_ctor_get(x_49, 1); +lean_inc(x_62); +if (lean_is_exclusive(x_49)) { + lean_ctor_release(x_49, 0); + lean_ctor_release(x_49, 1); + x_63 = x_49; +} else { + lean_dec_ref(x_49); + x_63 = lean_box(0); +} +if (lean_is_scalar(x_63)) { + x_64 = lean_alloc_ctor(1, 2, 0); +} else { + x_64 = x_63; +} +lean_ctor_set(x_64, 0, x_61); +lean_ctor_set(x_64, 1, x_62); +return x_64; +} } else { -lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; -lean_dec(x_33); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); +lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; +lean_dec(x_41); lean_dec(x_7); lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_44 = lean_ctor_get(x_39, 0); -lean_inc(x_44); -x_45 = lean_ctor_get(x_39, 1); -lean_inc(x_45); -if (lean_is_exclusive(x_39)) { - lean_ctor_release(x_39, 0); - lean_ctor_release(x_39, 1); - x_46 = x_39; +x_65 = lean_ctor_get(x_47, 0); +lean_inc(x_65); +x_66 = lean_ctor_get(x_47, 1); +lean_inc(x_66); +if (lean_is_exclusive(x_47)) { + lean_ctor_release(x_47, 0); + lean_ctor_release(x_47, 1); + x_67 = x_47; } else { - lean_dec_ref(x_39); - x_46 = lean_box(0); + lean_dec_ref(x_47); + x_67 = lean_box(0); } -if (lean_is_scalar(x_46)) { - x_47 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_67)) { + x_68 = lean_alloc_ctor(1, 2, 0); } else { - x_47 = x_46; -} -lean_ctor_set(x_47, 0, x_44); -lean_ctor_set(x_47, 1, x_45); -return x_47; -} + x_68 = x_67; } +lean_ctor_set(x_68, 0, x_65); +lean_ctor_set(x_68, 1, x_66); +return x_68; } } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; -x_12 = lean_ctor_get(x_4, 0); -lean_inc(x_12); -lean_dec(x_4); -x_13 = lean_ctor_get(x_12, 0); -lean_inc(x_13); -x_14 = lean_array_get_size(x_3); -x_15 = !lean_is_exclusive(x_9); -if (x_15 == 0) -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_9, 5); -x_17 = l_Lean_replaceRef(x_13, x_16); -lean_dec(x_16); -lean_dec(x_13); -lean_ctor_set(x_9, 5, 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_2); -x_18 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isInductiveFamily(x_14, x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_18) == 0) -{ -lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; lean_object* x_25; -x_19 = lean_ctor_get(x_18, 0); -lean_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_12, 8); -lean_inc(x_21); -lean_dec(x_12); -x_22 = lean_array_to_list(x_21); -x_23 = lean_box(0); -x_24 = lean_unbox(x_19); -lean_dec(x_19); -x_25 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2(x_1, x_2, x_3, x_24, x_22, x_23, x_5, x_6, x_7, x_8, x_9, x_10, x_20); -return x_25; } else { -uint8_t x_26; -lean_dec(x_9); -lean_dec(x_12); -lean_dec(x_10); -lean_dec(x_8); +uint8_t x_69; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_26 = !lean_is_exclusive(x_18); -if (x_26 == 0) +x_69 = !lean_is_exclusive(x_11); +if (x_69 == 0) { -return x_18; +return x_11; } else { -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_18, 0); -x_28 = lean_ctor_get(x_18, 1); -lean_inc(x_28); -lean_inc(x_27); -lean_dec(x_18); -x_29 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_29, 0, x_27); -lean_ctor_set(x_29, 1, x_28); -return x_29; +lean_object* x_70; lean_object* x_71; lean_object* x_72; +x_70 = lean_ctor_get(x_11, 0); +x_71 = lean_ctor_get(x_11, 1); +lean_inc(x_71); +lean_inc(x_70); +lean_dec(x_11); +x_72 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_72, 0, x_70); +lean_ctor_set(x_72, 1, x_71); +return x_72; } } } -else -{ -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; lean_object* x_42; uint8_t x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_30 = lean_ctor_get(x_9, 0); -x_31 = lean_ctor_get(x_9, 1); -x_32 = lean_ctor_get(x_9, 2); -x_33 = lean_ctor_get(x_9, 3); -x_34 = lean_ctor_get(x_9, 4); -x_35 = lean_ctor_get(x_9, 5); -x_36 = lean_ctor_get(x_9, 6); -x_37 = lean_ctor_get(x_9, 7); -x_38 = lean_ctor_get(x_9, 8); -x_39 = lean_ctor_get(x_9, 9); -x_40 = lean_ctor_get(x_9, 10); -x_41 = lean_ctor_get_uint8(x_9, sizeof(void*)*12); -x_42 = lean_ctor_get(x_9, 11); -x_43 = lean_ctor_get_uint8(x_9, sizeof(void*)*12 + 1); -lean_inc(x_42); -lean_inc(x_40); -lean_inc(x_39); -lean_inc(x_38); -lean_inc(x_37); -lean_inc(x_36); -lean_inc(x_35); -lean_inc(x_34); -lean_inc(x_33); -lean_inc(x_32); -lean_inc(x_31); -lean_inc(x_30); -lean_dec(x_9); -x_44 = l_Lean_replaceRef(x_13, x_35); -lean_dec(x_35); -lean_dec(x_13); -x_45 = lean_alloc_ctor(0, 12, 2); -lean_ctor_set(x_45, 0, x_30); -lean_ctor_set(x_45, 1, x_31); -lean_ctor_set(x_45, 2, x_32); -lean_ctor_set(x_45, 3, x_33); -lean_ctor_set(x_45, 4, x_34); -lean_ctor_set(x_45, 5, x_44); -lean_ctor_set(x_45, 6, x_36); -lean_ctor_set(x_45, 7, x_37); -lean_ctor_set(x_45, 8, x_38); -lean_ctor_set(x_45, 9, x_39); -lean_ctor_set(x_45, 10, x_40); -lean_ctor_set(x_45, 11, x_42); -lean_ctor_set_uint8(x_45, sizeof(void*)*12, x_41); -lean_ctor_set_uint8(x_45, sizeof(void*)*12 + 1, x_43); -lean_inc(x_10); -lean_inc(x_45); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_2); -x_46 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isInductiveFamily(x_14, x_2, x_5, x_6, x_7, x_8, x_45, x_10, x_11); -if (lean_obj_tag(x_46) == 0) -{ -lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; uint8_t x_52; lean_object* x_53; -x_47 = lean_ctor_get(x_46, 0); -lean_inc(x_47); -x_48 = lean_ctor_get(x_46, 1); -lean_inc(x_48); -lean_dec(x_46); -x_49 = lean_ctor_get(x_12, 8); -lean_inc(x_49); -lean_dec(x_12); -x_50 = lean_array_to_list(x_49); -x_51 = lean_box(0); -x_52 = lean_unbox(x_47); -lean_dec(x_47); -x_53 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2(x_1, x_2, x_3, x_52, x_50, x_51, x_5, x_6, x_7, x_8, x_45, x_10, x_48); -return x_53; } -else +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeader___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, 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_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; -lean_dec(x_45); -lean_dec(x_12); -lean_dec(x_10); +lean_object* x_10; +x_10 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeader___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_54 = lean_ctor_get(x_46, 0); -lean_inc(x_54); -x_55 = lean_ctor_get(x_46, 1); -lean_inc(x_55); -if (lean_is_exclusive(x_46)) { - lean_ctor_release(x_46, 0); - lean_ctor_release(x_46, 1); - x_56 = x_46; -} else { - lean_dec_ref(x_46); - x_56 = lean_box(0); -} -if (lean_is_scalar(x_56)) { - x_57 = lean_alloc_ctor(1, 2, 0); -} else { - x_57 = x_56; -} -lean_ctor_set(x_57, 0, x_54); -lean_ctor_set(x_57, 1, x_55); -return x_57; +return x_10; } } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls_loop___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_14 = lean_unsigned_to_nat(1u); +x_15 = lean_nat_add(x_1, x_14); +x_16 = lean_array_push(x_2, x_6); +x_17 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls_loop___rarg(x_3, x_4, x_5, x_15, x_16, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +return x_17; } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls_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, 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_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_13; uint8_t x_14; +x_13 = lean_array_get_size(x_2); +x_14 = lean_nat_dec_lt(x_4, x_13); +lean_dec(x_13); +if (x_14 == 0) +{ +lean_object* x_15; lean_dec(x_4); -x_7 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___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; +x_15 = lean_apply_9(x_1, x_3, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_16 = lean_array_fget(x_2, x_4); +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); +x_21 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls_loop___rarg___lambda__1___boxed), 13, 5); +lean_closure_set(x_21, 0, x_4); +lean_closure_set(x_21, 1, x_5); +lean_closure_set(x_21, 2, x_1); +lean_closure_set(x_21, 3, x_2); +lean_closure_set(x_21, 4, x_3); +x_22 = l_Lean_Elab_Term_withAuxDecl___rarg(x_19, x_20, x_18, x_21, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +return x_22; } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls_loop(lean_object* x_1) { _start: { -uint8_t x_3; lean_object* x_4; -x_3 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__1(x_1, x_2); -lean_dec(x_2); +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls_loop___rarg), 12, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls_loop___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; +x_14 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls_loop___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); lean_dec(x_1); -x_4 = lean_box(x_3); -return x_4; +return x_14; } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls___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: { -lean_object* x_11; -x_11 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +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); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -return x_11; +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_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_13); +x_16 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkTypeFor(x_13, x_4, x_5, 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; lean_object* x_21; lean_object* x_22; lean_object* x_23; size_t x_24; size_t x_25; lean_object* x_26; +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_13, 0); +lean_inc(x_19); +lean_dec(x_13); +x_20 = lean_ctor_get(x_19, 4); +lean_inc(x_20); +x_21 = lean_ctor_get(x_19, 3); +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_17); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_20); +lean_ctor_set(x_23, 1, x_22); +x_24 = 1; +x_25 = lean_usize_add(x_2, x_24); +x_26 = lean_array_uset(x_15, x_2, x_23); +x_2 = x_25; +x_3 = x_26; +x_10 = x_18; +goto _start; } -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { -_start: +else { -lean_object* x_15; -x_15 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +uint8_t x_28; +lean_dec(x_15); +lean_dec(x_13); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_2); -return x_15; -} -} -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___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_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_28 = !lean_is_exclusive(x_16); +if (x_28 == 0) { -lean_object* x_12; -x_12 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_1); -return x_12; -} +return x_16; } -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___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) { -_start: +else { -uint8_t x_14; lean_object* x_15; -x_14 = lean_unbox(x_5); -lean_dec(x_5); -x_15 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__5(x_1, x_2, x_3, x_4, x_14, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -return x_15; +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_16, 0); +x_30 = lean_ctor_get(x_16, 1); +lean_inc(x_30); +lean_inc(x_29); +lean_dec(x_16); +x_31 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_31, 0, x_29); +lean_ctor_set(x_31, 1, x_30); +return x_31; } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls___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: { -uint8_t x_14; lean_object* x_15; -x_14 = lean_unbox(x_4); -lean_dec(x_4); -x_15 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2(x_1, x_2, x_3, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -return x_15; +uint8_t x_13; +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; +x_14 = lean_ctor_get(x_10, 5); +x_15 = l_Lean_replaceRef(x_1, x_14); +lean_dec(x_14); +lean_ctor_set(x_10, 5, x_15); +x_16 = lean_unsigned_to_nat(0u); +x_17 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls_loop___rarg(x_2, x_3, x_4, x_16, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +return x_17; +} +else +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; lean_object* x_30; uint8_t x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_18 = lean_ctor_get(x_10, 0); +x_19 = lean_ctor_get(x_10, 1); +x_20 = lean_ctor_get(x_10, 2); +x_21 = lean_ctor_get(x_10, 3); +x_22 = lean_ctor_get(x_10, 4); +x_23 = lean_ctor_get(x_10, 5); +x_24 = lean_ctor_get(x_10, 6); +x_25 = lean_ctor_get(x_10, 7); +x_26 = lean_ctor_get(x_10, 8); +x_27 = lean_ctor_get(x_10, 9); +x_28 = lean_ctor_get(x_10, 10); +x_29 = lean_ctor_get_uint8(x_10, sizeof(void*)*12); +x_30 = lean_ctor_get(x_10, 11); +x_31 = lean_ctor_get_uint8(x_10, sizeof(void*)*12 + 1); +lean_inc(x_30); +lean_inc(x_28); +lean_inc(x_27); +lean_inc(x_26); +lean_inc(x_25); +lean_inc(x_24); +lean_inc(x_23); +lean_inc(x_22); +lean_inc(x_21); +lean_inc(x_20); +lean_inc(x_19); +lean_inc(x_18); +lean_dec(x_10); +x_32 = l_Lean_replaceRef(x_1, x_23); +lean_dec(x_23); +x_33 = lean_alloc_ctor(0, 12, 2); +lean_ctor_set(x_33, 0, x_18); +lean_ctor_set(x_33, 1, x_19); +lean_ctor_set(x_33, 2, x_20); +lean_ctor_set(x_33, 3, x_21); +lean_ctor_set(x_33, 4, x_22); +lean_ctor_set(x_33, 5, x_32); +lean_ctor_set(x_33, 6, x_24); +lean_ctor_set(x_33, 7, x_25); +lean_ctor_set(x_33, 8, x_26); +lean_ctor_set(x_33, 9, x_27); +lean_ctor_set(x_33, 10, x_28); +lean_ctor_set(x_33, 11, x_30); +lean_ctor_set_uint8(x_33, sizeof(void*)*12, x_29); +lean_ctor_set_uint8(x_33, sizeof(void*)*12 + 1, x_31); +x_34 = lean_unsigned_to_nat(0u); +x_35 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls_loop___rarg(x_2, x_3, x_4, x_34, x_5, x_6, x_7, x_8, x_9, x_33, x_11, x_12); +return x_35; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls___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_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; -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_is_exclusive(x_12); -if (x_13 == 0) +size_t x_10; size_t x_11; lean_object* x_12; +x_10 = lean_array_size(x_1); +x_11 = 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); +lean_inc(x_1); +x_12 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls___spec__1(x_10, x_11, x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_12) == 0) { -lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; -x_14 = lean_ctor_get(x_12, 0); -x_15 = lean_ctor_get(x_12, 1); -x_16 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(x_14, x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_15); -lean_dec(x_2); -x_17 = !lean_is_exclusive(x_16); +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_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_1); +x_16 = lean_unsigned_to_nat(0u); +x_17 = lean_nat_dec_lt(x_16, x_15); +lean_dec(x_15); if (x_17 == 0) { -lean_object* x_18; -x_18 = lean_ctor_get(x_16, 0); -lean_ctor_set(x_12, 1, x_18); -lean_ctor_set(x_12, 0, x_11); -lean_ctor_set_tag(x_16, 1); -lean_ctor_set(x_16, 0, x_12); -return x_16; +lean_object* x_28; lean_object* x_29; +lean_dec(x_1); +x_28 = l_Lean_Elab_Command_instInhabitedElabHeaderResult; +x_29 = l_outOfBounds___rarg(x_28); +x_18 = x_29; +goto block_27; } 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_object* x_30; +x_30 = lean_array_fget(x_1, x_16); +lean_dec(x_1); +x_18 = x_30; +goto block_27; +} +block_27: +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_19 = lean_ctor_get(x_18, 4); lean_inc(x_19); -lean_dec(x_16); -lean_ctor_set(x_12, 1, x_19); -lean_ctor_set(x_12, 0, x_11); -x_21 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_21, 0, x_12); -lean_ctor_set(x_21, 1, x_20); -return x_21; +x_20 = lean_ctor_get(x_18, 1); +lean_inc(x_20); +x_21 = lean_ctor_get(x_18, 2); +lean_inc(x_21); +x_22 = lean_ctor_get(x_18, 0); +lean_inc(x_22); +lean_dec(x_18); +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +lean_dec(x_22); +x_24 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__8___closed__1; +x_25 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls___rarg___lambda__1___boxed), 12, 5); +lean_closure_set(x_25, 0, x_23); +lean_closure_set(x_25, 1, x_2); +lean_closure_set(x_25, 2, x_13); +lean_closure_set(x_25, 3, x_19); +lean_closure_set(x_25, 4, x_24); +x_26 = l_Lean_Meta_withLCtx___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__3___rarg(x_20, x_21, x_25, x_3, x_4, x_5, x_6, x_7, x_8, x_14); +return x_26; } } 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; -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 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(x_22, x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_23); +uint8_t x_31; +lean_dec(x_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_25 = lean_ctor_get(x_24, 0); -lean_inc(x_25); -x_26 = lean_ctor_get(x_24, 1); -lean_inc(x_26); -if (lean_is_exclusive(x_24)) { - lean_ctor_release(x_24, 0); - lean_ctor_release(x_24, 1); - x_27 = x_24; -} else { - lean_dec_ref(x_24); - x_27 = lean_box(0); +lean_dec(x_1); +x_31 = !lean_is_exclusive(x_12); +if (x_31 == 0) +{ +return x_12; } -x_28 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_28, 0, x_11); -lean_ctor_set(x_28, 1, x_25); -if (lean_is_scalar(x_27)) { - x_29 = lean_alloc_ctor(1, 2, 0); -} else { - x_29 = x_27; - lean_ctor_set_tag(x_29, 1); +else +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; +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_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_ctor_set(x_29, 0, x_28); -lean_ctor_set(x_29, 1, x_26); -return x_29; } } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___lambda__1___closed__1() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls(lean_object* x_1) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("unexpected inductive type resulting type", 40, 40); -return x_1; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls___rarg), 9, 0); +return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___lambda__1___closed__2() { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls___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_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___lambda__1___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +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_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls___spec__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_Inductive_0__Lean_Elab_Command_getResultingUniverse___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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; +x_13 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_1); +return x_13; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isInductiveFamily___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; uint8_t x_12; lean_object* x_13; lean_object* x_14; +x_11 = lean_array_get_size(x_2); +x_12 = lean_nat_dec_lt(x_1, x_11); +lean_dec(x_11); +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_10); +return x_14; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isInductiveFamily(lean_object* x_1, lean_object* x_2, lean_object* x_3, 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; @@ -10363,1101 +11429,1210 @@ lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_10 = l_Lean_Meta_whnfD(x_2, x_5, x_6, x_7, x_8, x_9); +x_10 = lean_infer_type(x_2, x_5, x_6, x_7, x_8, x_9); if (lean_obj_tag(x_10) == 0) { -lean_object* x_11; +lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; lean_object* x_15; x_11 = lean_ctor_get(x_10, 0); lean_inc(x_11); -if (lean_obj_tag(x_11) == 3) +x_12 = lean_ctor_get(x_10, 1); +lean_inc(x_12); +lean_dec(x_10); +x_13 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isInductiveFamily___lambda__1___boxed), 10, 1); +lean_closure_set(x_13, 0, x_1); +x_14 = 0; +x_15 = l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___spec__1___rarg(x_11, x_13, x_14, x_3, x_4, x_5, x_6, x_7, x_8, x_12); +return x_15; +} +else { -uint8_t x_12; +uint8_t x_16; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); -x_12 = !lean_is_exclusive(x_10); -if (x_12 == 0) +lean_dec(x_1); +x_16 = !lean_is_exclusive(x_10); +if (x_16 == 0) { -lean_object* x_13; lean_object* x_14; -x_13 = lean_ctor_get(x_10, 0); -lean_dec(x_13); -x_14 = lean_ctor_get(x_11, 0); -lean_inc(x_14); -lean_dec(x_11); -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); -x_16 = lean_ctor_get(x_11, 0); -lean_inc(x_16); -lean_dec(x_11); -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_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +lean_object* x_17; lean_object* x_18; lean_object* x_19; +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_10); -x_19 = l_Lean_indentExpr(x_11); -x_20 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___lambda__1___closed__2; -x_21 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_21, 0, x_20); -lean_ctor_set(x_21, 1, x_19); -x_22 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5; -x_23 = lean_alloc_ctor(7, 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_Inductive_0__Lean_Elab_Command_getResultingUniverse___spec__1(x_23, x_3, x_4, x_5, x_6, x_7, x_8, x_18); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -return x_24; +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; } } -else +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isInductiveFamily___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_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_25; +lean_object* x_11; +x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isInductiveFamily___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); -x_25 = !lean_is_exclusive(x_10); -if (x_25 == 0) +lean_dec(x_2); +lean_dec(x_1); +return x_11; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getArrowBinderNames_go(lean_object* x_1, lean_object* x_2) { +_start: { -return x_10; +switch (lean_obj_tag(x_1)) { +case 7: +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_3 = lean_ctor_get(x_1, 0); +lean_inc(x_3); +x_4 = lean_ctor_get(x_1, 2); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_array_push(x_2, x_3); +x_1 = x_4; +x_2 = x_5; +goto _start; } -else +case 10: { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_10, 0); -x_27 = lean_ctor_get(x_10, 1); -lean_inc(x_27); -lean_inc(x_26); -lean_dec(x_10); -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_7; +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +lean_dec(x_1); +x_1 = x_7; +goto _start; +} +default: +{ +lean_dec(x_1); +return x_2; } } } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___closed__1() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getArrowBinderNames(lean_object* x_1) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("unexpected empty inductive declaration", 38, 38); -return x_1; +lean_object* x_2; lean_object* x_3; +x_2 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__8___closed__1; +x_3 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getArrowBinderNames_go(x_1, x_2); +return x_3; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___closed__2() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceArrowBinderNames_go(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); +lean_object* x_4; uint8_t x_5; +x_4 = lean_array_get_size(x_1); +x_5 = lean_nat_dec_lt(x_3, x_4); +lean_dec(x_4); +if (x_5 == 0) +{ return x_2; } -} -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___closed__3() { -_start: +else { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___lambda__1___boxed), 9, 0); -return x_1; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse(lean_object* x_1, lean_object* x_2, lean_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_2) == 7) { -if (lean_obj_tag(x_1) == 0) +lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; uint8_t x_10; +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_ctor_get_uint8(x_2, sizeof(void*)*3 + 8); +lean_dec(x_2); +x_10 = l_Lean_Name_hasMacroScopes(x_6); +if (x_10 == 0) { -lean_object* x_9; lean_object* x_10; -x_9 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___closed__2; -x_10 = l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___spec__1(x_9, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_7); +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 = lean_nat_add(x_3, x_11); +x_13 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceArrowBinderNames_go(x_1, x_8, x_12); +lean_dec(x_12); +x_14 = l_Lean_Expr_forallE___override(x_6, x_7, x_13, x_9); +return x_14; +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -return x_10; +x_15 = lean_array_fget(x_1, x_3); +x_16 = lean_unsigned_to_nat(1u); +x_17 = lean_nat_add(x_3, x_16); +x_18 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceArrowBinderNames_go(x_1, x_8, x_17); +lean_dec(x_17); +x_19 = l_Lean_Expr_forallE___override(x_15, x_7, x_18, x_9); +return x_19; +} } else { -lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; lean_object* x_15; -x_11 = lean_ctor_get(x_1, 0); -lean_inc(x_11); -lean_dec(x_1); -x_12 = lean_ctor_get(x_11, 1); -lean_inc(x_12); -lean_dec(x_11); -x_13 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___closed__3; -x_14 = 0; -x_15 = l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___spec__1___rarg(x_12, x_13, x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -return x_15; +return x_2; } } } -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceArrowBinderNames_go___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_9; -x_9 = l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___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_object* x_4; +x_4 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceArrowBinderNames_go(x_1, x_2, x_3); lean_dec(x_3); -return x_9; +lean_dec(x_1); +return x_4; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_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_Inductive_0__Lean_Elab_Command_replaceArrowBinderNames(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_10; -x_10 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___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_1); -return x_10; +lean_object* x_3; lean_object* x_4; +x_3 = lean_unsigned_to_nat(0u); +x_4 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceArrowBinderNames_go(x_2, x_1, x_3); +return x_4; } } -LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_shouldInferResultUniverse___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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceArrowBinderNames___boxed(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; -x_9 = lean_st_ref_get(x_5, 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, 0); -lean_inc(x_12); -lean_dec(x_10); -x_13 = lean_instantiate_level_mvars(x_12, x_1); -x_14 = lean_ctor_get(x_13, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_13, 1); -lean_inc(x_15); -lean_dec(x_13); -x_16 = lean_st_ref_take(x_5, x_11); -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_16, 1); -lean_inc(x_18); -lean_dec(x_16); -x_19 = !lean_is_exclusive(x_17); -if (x_19 == 0) -{ -lean_object* x_20; lean_object* x_21; uint8_t x_22; -x_20 = lean_ctor_get(x_17, 0); -lean_dec(x_20); -lean_ctor_set(x_17, 0, x_14); -x_21 = lean_st_ref_set(x_5, x_17, x_18); -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_15); -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_15); -lean_ctor_set(x_25, 1, x_24); -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_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_26 = lean_ctor_get(x_17, 1); -x_27 = lean_ctor_get(x_17, 2); -x_28 = lean_ctor_get(x_17, 3); -x_29 = lean_ctor_get(x_17, 4); -lean_inc(x_29); -lean_inc(x_28); -lean_inc(x_27); -lean_inc(x_26); -lean_dec(x_17); -x_30 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_30, 0, x_14); -lean_ctor_set(x_30, 1, x_26); -lean_ctor_set(x_30, 2, x_27); -lean_ctor_set(x_30, 3, x_28); -lean_ctor_set(x_30, 4, x_29); -x_31 = lean_st_ref_set(x_5, x_30, x_18); -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; -} else { - lean_dec_ref(x_31); - x_33 = lean_box(0); -} -if (lean_is_scalar(x_33)) { - x_34 = lean_alloc_ctor(0, 2, 0); -} else { - x_34 = x_33; -} -lean_ctor_set(x_34, 0, x_15); -lean_ctor_set(x_34, 1, x_32); -return x_34; -} +lean_object* x_3; +x_3 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceArrowBinderNames(x_1, x_2); +lean_dec(x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_shouldInferResultUniverse___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_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__1(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4) { _start: { -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_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_is_exclusive(x_12); -if (x_13 == 0) +uint8_t x_5; +x_5 = lean_usize_dec_eq(x_3, x_4); +if (x_5 == 0) { -lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; -x_14 = lean_ctor_get(x_12, 0); -x_15 = lean_ctor_get(x_12, 1); -x_16 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(x_14, x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_15); -lean_dec(x_2); -x_17 = !lean_is_exclusive(x_16); -if (x_17 == 0) +lean_object* x_6; lean_object* x_7; uint8_t x_8; +x_6 = lean_array_uget(x_2, x_3); +x_7 = l_Lean_Expr_fvarId_x21(x_6); +lean_dec(x_6); +x_8 = lean_name_eq(x_7, x_1); +lean_dec(x_7); +if (x_8 == 0) { -lean_object* x_18; -x_18 = lean_ctor_get(x_16, 0); -lean_ctor_set(x_12, 1, x_18); -lean_ctor_set(x_12, 0, x_11); -lean_ctor_set_tag(x_16, 1); -lean_ctor_set(x_16, 0, x_12); -return x_16; +size_t x_9; size_t x_10; +x_9 = 1; +x_10 = lean_usize_add(x_3, x_9); +x_3 = x_10; +goto _start; } 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_12, 1, x_19); -lean_ctor_set(x_12, 0, x_11); -x_21 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_21, 0, x_12); -lean_ctor_set(x_21, 1, x_20); -return x_21; +uint8_t x_12; +x_12 = 1; +return x_12; } } 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; -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 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(x_22, x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_23); -lean_dec(x_2); -x_25 = lean_ctor_get(x_24, 0); -lean_inc(x_25); -x_26 = lean_ctor_get(x_24, 1); -lean_inc(x_26); -if (lean_is_exclusive(x_24)) { - lean_ctor_release(x_24, 0); - lean_ctor_release(x_24, 1); - x_27 = x_24; -} else { - lean_dec_ref(x_24); - x_27 = lean_box(0); -} -x_28 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_28, 0, x_11); -lean_ctor_set(x_28, 1, x_25); -if (lean_is_scalar(x_27)) { - x_29 = lean_alloc_ctor(1, 2, 0); -} else { - x_29 = x_27; - lean_ctor_set_tag(x_29, 1); -} -lean_ctor_set(x_29, 0, x_28); -lean_ctor_set(x_29, 1, x_26); -return x_29; -} -} +uint8_t x_13; +x_13 = 0; +return x_13; } -static lean_object* _init_l_Lean_Elab_Command_shouldInferResultUniverse___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("cannot infer resulting universe level of inductive datatype, given level contains metavariables ", 96, 96); -return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_shouldInferResultUniverse___closed__2() { +static lean_object* _init_l_Lean_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__2___closed__1() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_shouldInferResultUniverse___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_unsigned_to_nat(10u); +x_2 = lean_unsigned_to_nat(1u); +x_3 = l_Nat_nextPowerOfTwo_go(x_1, x_2, lean_box(0)); +return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_shouldInferResultUniverse___closed__3() { +static lean_object* _init_l_Lean_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__2___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked(", provide universe explicitly", 29, 29); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__2___closed__1; +x_3 = lean_mk_array(x_2, x_1); +return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_shouldInferResultUniverse___closed__4() { +static lean_object* _init_l_Lean_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__2___closed__3() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_shouldInferResultUniverse___closed__3; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_unsigned_to_nat(0u); +x_2 = l_Lean_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___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_EXPORT lean_object* l_Lean_Elab_Command_shouldInferResultUniverse(lean_object* x_1, lean_object* x_2, lean_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_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___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; uint8_t x_10; -x_9 = l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_shouldInferResultUniverse___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -x_10 = !lean_is_exclusive(x_9); -if (x_10 == 0) -{ -lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_11 = lean_ctor_get(x_9, 0); -x_12 = lean_ctor_get(x_9, 1); -x_13 = l_Lean_Level_hasMVar(x_11); -if (x_13 == 0) -{ -lean_object* x_14; -lean_dec(x_11); -lean_dec(x_2); -x_14 = lean_box(0); -lean_ctor_set(x_9, 0, x_14); -return x_9; -} -else +if (lean_obj_tag(x_1) == 0) { -lean_object* x_15; -x_15 = l_Lean_Level_getLevelOffset(x_11); -if (lean_obj_tag(x_15) == 5) +lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_9 = lean_ctor_get(x_1, 3); +lean_inc(x_9); +lean_dec(x_1); +x_10 = lean_st_ref_get(x_5, x_8); +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) { -lean_object* x_16; lean_object* x_17; -lean_dec(x_11); -lean_dec(x_2); -x_16 = lean_ctor_get(x_15, 0); -lean_inc(x_16); -lean_dec(x_15); -x_17 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_17, 0, x_16); -lean_ctor_set(x_9, 0, x_17); -return x_9; -} -else +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_10, 0); +x_13 = lean_ctor_get(x_10, 1); +x_14 = lean_ctor_get(x_12, 0); +lean_inc(x_14); +lean_dec(x_12); +x_15 = l_Lean_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__2___closed__3; +lean_inc(x_14); +lean_ctor_set(x_10, 1, x_14); +lean_ctor_set(x_10, 0, x_15); +x_16 = l_Lean_Expr_hasFVar(x_9); +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; lean_object* x_24; -lean_dec(x_15); -lean_free_object(x_9); -x_18 = l_Lean_Expr_sort___override(x_11); -x_19 = l_Lean_MessageData_ofExpr(x_18); -x_20 = l_Lean_Elab_Command_shouldInferResultUniverse___closed__2; -x_21 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_21, 0, x_20); -lean_ctor_set(x_21, 1, x_19); -x_22 = l_Lean_Elab_Command_shouldInferResultUniverse___closed__4; -x_23 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_23, 0, x_21); -lean_ctor_set(x_23, 1, x_22); -x_24 = l_Lean_throwError___at_Lean_Elab_Command_shouldInferResultUniverse___spec__2(x_23, x_2, x_3, x_4, x_5, x_6, x_7, x_12); -return x_24; -} -} -} -else +uint8_t x_17; +x_17 = l_Lean_Expr_hasMVar(x_9); +if (x_17 == 0) { -lean_object* x_25; lean_object* x_26; uint8_t x_27; -x_25 = lean_ctor_get(x_9, 0); -x_26 = lean_ctor_get(x_9, 1); -lean_inc(x_26); -lean_inc(x_25); +lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +lean_dec(x_10); lean_dec(x_9); -x_27 = l_Lean_Level_hasMVar(x_25); -if (x_27 == 0) -{ -lean_object* x_28; lean_object* x_29; -lean_dec(x_25); +lean_dec(x_3); lean_dec(x_2); -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_26); -return x_29; -} -else +x_18 = lean_st_ref_take(x_5, 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 = !lean_is_exclusive(x_19); +if (x_21 == 0) { -lean_object* x_30; -x_30 = l_Lean_Level_getLevelOffset(x_25); -if (lean_obj_tag(x_30) == 5) +lean_object* x_22; lean_object* x_23; uint8_t x_24; +x_22 = lean_ctor_get(x_19, 0); +lean_dec(x_22); +lean_ctor_set(x_19, 0, x_14); +x_23 = lean_st_ref_set(x_5, x_19, x_20); +x_24 = !lean_is_exclusive(x_23); +if (x_24 == 0) { -lean_object* x_31; lean_object* x_32; lean_object* x_33; +lean_object* x_25; uint8_t x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_23, 0); lean_dec(x_25); -lean_dec(x_2); -x_31 = lean_ctor_get(x_30, 0); -lean_inc(x_31); -lean_dec(x_30); -x_32 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_32, 0, x_31); -x_33 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_33, 0, x_32); -lean_ctor_set(x_33, 1, x_26); -return x_33; +x_26 = 0; +x_27 = lean_box(x_26); +lean_ctor_set(x_23, 0, x_27); +return x_23; } 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_dec(x_30); -x_34 = l_Lean_Expr_sort___override(x_25); -x_35 = l_Lean_MessageData_ofExpr(x_34); -x_36 = l_Lean_Elab_Command_shouldInferResultUniverse___closed__2; -x_37 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_37, 0, x_36); -lean_ctor_set(x_37, 1, x_35); -x_38 = l_Lean_Elab_Command_shouldInferResultUniverse___closed__4; -x_39 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_39, 0, x_37); -lean_ctor_set(x_39, 1, x_38); -x_40 = l_Lean_throwError___at_Lean_Elab_Command_shouldInferResultUniverse___spec__2(x_39, x_2, x_3, x_4, x_5, x_6, x_7, x_26); -return x_40; -} -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_shouldInferResultUniverse___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_instantiateLevelMVars___at_Lean_Elab_Command_shouldInferResultUniverse___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_28; uint8_t x_29; lean_object* x_30; lean_object* x_31; +x_28 = lean_ctor_get(x_23, 1); +lean_inc(x_28); +lean_dec(x_23); +x_29 = 0; +x_30 = lean_box(x_29); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_30); +lean_ctor_set(x_31, 1, x_28); +return x_31; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_shouldInferResultUniverse___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) { -_start: +else { -lean_object* x_9; -x_9 = l_Lean_throwError___at_Lean_Elab_Command_shouldInferResultUniverse___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -return x_9; +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; lean_object* x_41; lean_object* x_42; +x_32 = lean_ctor_get(x_19, 1); +x_33 = lean_ctor_get(x_19, 2); +x_34 = lean_ctor_get(x_19, 3); +x_35 = lean_ctor_get(x_19, 4); +lean_inc(x_35); +lean_inc(x_34); +lean_inc(x_33); +lean_inc(x_32); +lean_dec(x_19); +x_36 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_36, 0, x_14); +lean_ctor_set(x_36, 1, x_32); +lean_ctor_set(x_36, 2, x_33); +lean_ctor_set(x_36, 3, x_34); +lean_ctor_set(x_36, 4, x_35); +x_37 = lean_st_ref_set(x_5, x_36, x_20); +x_38 = lean_ctor_get(x_37, 1); +lean_inc(x_38); +if (lean_is_exclusive(x_37)) { + lean_ctor_release(x_37, 0); + lean_ctor_release(x_37, 1); + x_39 = x_37; +} else { + lean_dec_ref(x_37); + x_39 = lean_box(0); } +x_40 = 0; +x_41 = lean_box(x_40); +if (lean_is_scalar(x_39)) { + x_42 = lean_alloc_ctor(0, 2, 0); +} else { + x_42 = x_39; } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_shouldInferResultUniverse___boxed(lean_object* x_1, lean_object* x_2, lean_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_Command_shouldInferResultUniverse(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_ctor_set(x_42, 0, x_41); +lean_ctor_set(x_42, 1, x_38); +return x_42; } } -LEAN_EXPORT uint8_t l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27___spec__1(lean_object* x_1, lean_object* x_2) { -_start: +else { -if (lean_obj_tag(x_1) == 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_dec(x_14); +x_43 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit(x_2, x_3, x_9, x_10); +x_44 = lean_ctor_get(x_43, 1); +lean_inc(x_44); +x_45 = lean_ctor_get(x_43, 0); +lean_inc(x_45); +lean_dec(x_43); +x_46 = lean_ctor_get(x_44, 1); +lean_inc(x_46); +lean_dec(x_44); +x_47 = lean_st_ref_take(x_5, x_13); +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_is_exclusive(x_48); +if (x_50 == 0) { -if (lean_obj_tag(x_2) == 0) +lean_object* x_51; lean_object* x_52; uint8_t x_53; +x_51 = lean_ctor_get(x_48, 0); +lean_dec(x_51); +lean_ctor_set(x_48, 0, x_46); +x_52 = lean_st_ref_set(x_5, x_48, x_49); +x_53 = !lean_is_exclusive(x_52); +if (x_53 == 0) { -uint8_t x_3; -x_3 = 1; -return x_3; +lean_object* x_54; +x_54 = lean_ctor_get(x_52, 0); +lean_dec(x_54); +lean_ctor_set(x_52, 0, x_45); +return x_52; } else { -uint8_t x_4; -x_4 = 0; -return x_4; -} +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_45); +lean_ctor_set(x_56, 1, x_55); +return x_56; } -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; uint8_t x_8; -x_6 = lean_ctor_get(x_1, 0); -x_7 = lean_ctor_get(x_2, 0); -x_8 = lean_name_eq(x_6, x_7); -return x_8; -} +lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_57 = lean_ctor_get(x_48, 1); +x_58 = lean_ctor_get(x_48, 2); +x_59 = lean_ctor_get(x_48, 3); +x_60 = lean_ctor_get(x_48, 4); +lean_inc(x_60); +lean_inc(x_59); +lean_inc(x_58); +lean_inc(x_57); +lean_dec(x_48); +x_61 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_61, 0, x_46); +lean_ctor_set(x_61, 1, x_57); +lean_ctor_set(x_61, 2, x_58); +lean_ctor_set(x_61, 3, x_59); +lean_ctor_set(x_61, 4, x_60); +x_62 = lean_st_ref_set(x_5, x_61, x_49); +x_63 = lean_ctor_get(x_62, 1); +lean_inc(x_63); +if (lean_is_exclusive(x_62)) { + lean_ctor_release(x_62, 0); + lean_ctor_release(x_62, 1); + x_64 = x_62; +} else { + lean_dec_ref(x_62); + x_64 = lean_box(0); } +if (lean_is_scalar(x_64)) { + x_65 = lean_alloc_ctor(0, 2, 0); +} else { + x_65 = x_64; } +lean_ctor_set(x_65, 0, x_45); +lean_ctor_set(x_65, 1, x_63); +return x_65; } -LEAN_EXPORT uint8_t l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27___lambda__1(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; uint8_t x_4; -x_3 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_3, 0, x_2); -x_4 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27___spec__1(x_1, x_3); -lean_dec(x_3); -return x_4; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_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) { -_start: +else { -lean_object* x_10; lean_object* x_11; -x_10 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27___lambda__1___boxed), 2, 1); -lean_closure_set(x_10, 0, x_1); -x_11 = l_Lean_Elab_Term_levelMVarToParam(x_2, x_10, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_11; -} +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_dec(x_14); +x_66 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit(x_2, x_3, x_9, x_10); +x_67 = lean_ctor_get(x_66, 1); +lean_inc(x_67); +x_68 = lean_ctor_get(x_66, 0); +lean_inc(x_68); +lean_dec(x_66); +x_69 = lean_ctor_get(x_67, 1); +lean_inc(x_69); +lean_dec(x_67); +x_70 = lean_st_ref_take(x_5, x_13); +x_71 = lean_ctor_get(x_70, 0); +lean_inc(x_71); +x_72 = lean_ctor_get(x_70, 1); +lean_inc(x_72); +lean_dec(x_70); +x_73 = !lean_is_exclusive(x_71); +if (x_73 == 0) +{ +lean_object* x_74; lean_object* x_75; uint8_t x_76; +x_74 = lean_ctor_get(x_71, 0); +lean_dec(x_74); +lean_ctor_set(x_71, 0, x_69); +x_75 = lean_st_ref_set(x_5, x_71, x_72); +x_76 = !lean_is_exclusive(x_75); +if (x_76 == 0) +{ +lean_object* x_77; +x_77 = lean_ctor_get(x_75, 0); +lean_dec(x_77); +lean_ctor_set(x_75, 0, x_68); +return x_75; } -LEAN_EXPORT lean_object* l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27___spec__1___boxed(lean_object* x_1, lean_object* x_2) { -_start: +else { -uint8_t x_3; lean_object* x_4; -x_3 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27___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_78; lean_object* x_79; +x_78 = lean_ctor_get(x_75, 1); +lean_inc(x_78); +lean_dec(x_75); +x_79 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_79, 0, x_68); +lean_ctor_set(x_79, 1, x_78); +return x_79; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { -_start: +else { -uint8_t x_3; lean_object* x_4; -x_3 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27___lambda__1(x_1, x_2); -lean_dec(x_1); -x_4 = lean_box(x_3); -return x_4; +lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; +x_80 = lean_ctor_get(x_71, 1); +x_81 = lean_ctor_get(x_71, 2); +x_82 = lean_ctor_get(x_71, 3); +x_83 = lean_ctor_get(x_71, 4); +lean_inc(x_83); +lean_inc(x_82); +lean_inc(x_81); +lean_inc(x_80); +lean_dec(x_71); +x_84 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_84, 0, x_69); +lean_ctor_set(x_84, 1, x_80); +lean_ctor_set(x_84, 2, x_81); +lean_ctor_set(x_84, 3, x_82); +lean_ctor_set(x_84, 4, x_83); +x_85 = lean_st_ref_set(x_5, x_84, x_72); +x_86 = lean_ctor_get(x_85, 1); +lean_inc(x_86); +if (lean_is_exclusive(x_85)) { + lean_ctor_release(x_85, 0); + lean_ctor_release(x_85, 1); + x_87 = x_85; +} else { + lean_dec_ref(x_85); + x_87 = lean_box(0); } +if (lean_is_scalar(x_87)) { + x_88 = lean_alloc_ctor(0, 2, 0); +} else { + x_88 = x_87; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_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) { -_start: -{ -lean_object* x_10; -x_10 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -return x_10; +lean_ctor_set(x_88, 0, x_68); +lean_ctor_set(x_88, 1, x_86); +return x_88; } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam___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: -{ -if (lean_obj_tag(x_2) == 0) -{ -lean_object* x_11; lean_object* x_12; -lean_dec(x_1); -x_11 = l_List_reverse___rarg(x_3); -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; } else { -uint8_t x_13; -x_13 = !lean_is_exclusive(x_2); -if (x_13 == 0) -{ -lean_object* x_14; uint8_t x_15; -x_14 = lean_ctor_get(x_2, 0); -x_15 = !lean_is_exclusive(x_14); -if (x_15 == 0) +lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; uint8_t x_94; +x_89 = lean_ctor_get(x_10, 0); +x_90 = lean_ctor_get(x_10, 1); +lean_inc(x_90); +lean_inc(x_89); +lean_dec(x_10); +x_91 = lean_ctor_get(x_89, 0); +lean_inc(x_91); +lean_dec(x_89); +x_92 = l_Lean_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__2___closed__3; +lean_inc(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_91); +x_94 = l_Lean_Expr_hasFVar(x_9); +if (x_94 == 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_2, 1); -x_17 = lean_ctor_get(x_14, 1); -lean_inc(x_1); -x_18 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27(x_1, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -x_19 = lean_ctor_get(x_18, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_18, 1); -lean_inc(x_20); -lean_dec(x_18); -lean_ctor_set(x_14, 1, x_19); -lean_ctor_set(x_2, 1, x_3); +uint8_t x_95; +x_95 = l_Lean_Expr_hasMVar(x_9); +if (x_95 == 0) { -lean_object* _tmp_1 = x_16; -lean_object* _tmp_2 = x_2; -lean_object* _tmp_9 = x_20; -x_2 = _tmp_1; -x_3 = _tmp_2; -x_10 = _tmp_9; +lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; uint8_t x_108; lean_object* x_109; lean_object* x_110; +lean_dec(x_93); +lean_dec(x_9); +lean_dec(x_3); +lean_dec(x_2); +x_96 = lean_st_ref_take(x_5, x_90); +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_ctor_get(x_97, 1); +lean_inc(x_99); +x_100 = lean_ctor_get(x_97, 2); +lean_inc(x_100); +x_101 = lean_ctor_get(x_97, 3); +lean_inc(x_101); +x_102 = lean_ctor_get(x_97, 4); +lean_inc(x_102); +if (lean_is_exclusive(x_97)) { + lean_ctor_release(x_97, 0); + lean_ctor_release(x_97, 1); + lean_ctor_release(x_97, 2); + lean_ctor_release(x_97, 3); + lean_ctor_release(x_97, 4); + x_103 = x_97; +} else { + lean_dec_ref(x_97); + x_103 = lean_box(0); } -goto _start; +if (lean_is_scalar(x_103)) { + x_104 = lean_alloc_ctor(0, 5, 0); +} else { + x_104 = x_103; +} +lean_ctor_set(x_104, 0, x_91); +lean_ctor_set(x_104, 1, x_99); +lean_ctor_set(x_104, 2, x_100); +lean_ctor_set(x_104, 3, x_101); +lean_ctor_set(x_104, 4, x_102); +x_105 = lean_st_ref_set(x_5, x_104, x_98); +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 = 0; +x_109 = lean_box(x_108); +if (lean_is_scalar(x_107)) { + x_110 = lean_alloc_ctor(0, 2, 0); +} else { + x_110 = x_107; +} +lean_ctor_set(x_110, 0, x_109); +lean_ctor_set(x_110, 1, x_106); +return x_110; } 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; -x_22 = lean_ctor_get(x_2, 1); -x_23 = lean_ctor_get(x_14, 0); -x_24 = lean_ctor_get(x_14, 1); -lean_inc(x_24); -lean_inc(x_23); -lean_dec(x_14); -lean_inc(x_1); -x_25 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27(x_1, x_24, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -x_26 = lean_ctor_get(x_25, 0); -lean_inc(x_26); -x_27 = lean_ctor_get(x_25, 1); -lean_inc(x_27); -lean_dec(x_25); -x_28 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_28, 0, x_23); -lean_ctor_set(x_28, 1, x_26); -lean_ctor_set(x_2, 1, x_3); -lean_ctor_set(x_2, 0, x_28); -{ -lean_object* _tmp_1 = x_22; -lean_object* _tmp_2 = x_2; -lean_object* _tmp_9 = x_27; -x_2 = _tmp_1; -x_3 = _tmp_2; -x_10 = _tmp_9; +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_dec(x_91); +x_111 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit(x_2, x_3, x_9, x_93); +x_112 = lean_ctor_get(x_111, 1); +lean_inc(x_112); +x_113 = lean_ctor_get(x_111, 0); +lean_inc(x_113); +lean_dec(x_111); +x_114 = lean_ctor_get(x_112, 1); +lean_inc(x_114); +lean_dec(x_112); +x_115 = lean_st_ref_take(x_5, x_90); +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, 1); +lean_inc(x_118); +x_119 = lean_ctor_get(x_116, 2); +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); +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); + x_122 = x_116; +} else { + lean_dec_ref(x_116); + x_122 = lean_box(0); } -goto _start; +if (lean_is_scalar(x_122)) { + x_123 = lean_alloc_ctor(0, 5, 0); +} else { + x_123 = x_122; +} +lean_ctor_set(x_123, 0, x_114); +lean_ctor_set(x_123, 1, x_118); +lean_ctor_set(x_123, 2, x_119); +lean_ctor_set(x_123, 3, x_120); +lean_ctor_set(x_123, 4, x_121); +x_124 = lean_st_ref_set(x_5, x_123, x_117); +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_124); + x_126 = lean_box(0); +} +if (lean_is_scalar(x_126)) { + x_127 = lean_alloc_ctor(0, 2, 0); +} else { + x_127 = x_126; +} +lean_ctor_set(x_127, 0, x_113); +lean_ctor_set(x_127, 1, x_125); +return x_127; } } else { -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_30 = lean_ctor_get(x_2, 0); -x_31 = lean_ctor_get(x_2, 1); -lean_inc(x_31); -lean_inc(x_30); -lean_dec(x_2); -x_32 = lean_ctor_get(x_30, 0); -lean_inc(x_32); -x_33 = lean_ctor_get(x_30, 1); -lean_inc(x_33); -if (lean_is_exclusive(x_30)) { - lean_ctor_release(x_30, 0); - lean_ctor_release(x_30, 1); - x_34 = x_30; +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_dec(x_91); +x_128 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit(x_2, x_3, x_9, x_93); +x_129 = lean_ctor_get(x_128, 1); +lean_inc(x_129); +x_130 = lean_ctor_get(x_128, 0); +lean_inc(x_130); +lean_dec(x_128); +x_131 = lean_ctor_get(x_129, 1); +lean_inc(x_131); +lean_dec(x_129); +x_132 = lean_st_ref_take(x_5, x_90); +x_133 = lean_ctor_get(x_132, 0); +lean_inc(x_133); +x_134 = lean_ctor_get(x_132, 1); +lean_inc(x_134); +lean_dec(x_132); +x_135 = lean_ctor_get(x_133, 1); +lean_inc(x_135); +x_136 = lean_ctor_get(x_133, 2); +lean_inc(x_136); +x_137 = lean_ctor_get(x_133, 3); +lean_inc(x_137); +x_138 = lean_ctor_get(x_133, 4); +lean_inc(x_138); +if (lean_is_exclusive(x_133)) { + lean_ctor_release(x_133, 0); + lean_ctor_release(x_133, 1); + lean_ctor_release(x_133, 2); + lean_ctor_release(x_133, 3); + lean_ctor_release(x_133, 4); + x_139 = x_133; } else { - lean_dec_ref(x_30); - x_34 = lean_box(0); + lean_dec_ref(x_133); + x_139 = lean_box(0); } -lean_inc(x_1); -x_35 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27(x_1, x_33, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -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); -if (lean_is_scalar(x_34)) { - x_38 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_139)) { + x_140 = lean_alloc_ctor(0, 5, 0); } else { - x_38 = x_34; + x_140 = x_139; } -lean_ctor_set(x_38, 0, x_32); -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_2 = x_31; -x_3 = x_39; -x_10 = x_37; -goto _start; +lean_ctor_set(x_140, 0, x_131); +lean_ctor_set(x_140, 1, x_135); +lean_ctor_set(x_140, 2, x_136); +lean_ctor_set(x_140, 3, x_137); +lean_ctor_set(x_140, 4, x_138); +x_141 = lean_st_ref_set(x_5, x_140, x_134); +x_142 = lean_ctor_get(x_141, 1); +lean_inc(x_142); +if (lean_is_exclusive(x_141)) { + lean_ctor_release(x_141, 0); + lean_ctor_release(x_141, 1); + x_143 = x_141; +} else { + lean_dec_ref(x_141); + x_143 = lean_box(0); } +if (lean_is_scalar(x_143)) { + x_144 = lean_alloc_ctor(0, 2, 0); +} else { + x_144 = x_143; } +lean_ctor_set(x_144, 0, x_130); +lean_ctor_set(x_144, 1, x_142); +return x_144; } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam___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: -{ -if (lean_obj_tag(x_2) == 0) -{ -lean_object* x_11; lean_object* x_12; -lean_dec(x_1); -x_11 = l_List_reverse___rarg(x_3); -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; } else { -uint8_t x_13; -x_13 = !lean_is_exclusive(x_2); -if (x_13 == 0) +lean_object* x_145; lean_object* x_146; lean_object* x_147; uint8_t x_148; +x_145 = lean_ctor_get(x_1, 3); +lean_inc(x_145); +x_146 = lean_ctor_get(x_1, 4); +lean_inc(x_146); +lean_dec(x_1); +x_147 = lean_st_ref_get(x_5, x_8); +x_148 = !lean_is_exclusive(x_147); +if (x_148 == 0) { -lean_object* x_14; uint8_t x_15; -x_14 = lean_ctor_get(x_2, 0); -x_15 = !lean_is_exclusive(x_14); -if (x_15 == 0) +lean_object* x_149; lean_object* x_150; lean_object* x_151; uint8_t x_152; lean_object* x_153; uint8_t x_178; lean_object* x_179; lean_object* x_192; uint8_t x_193; +x_149 = lean_ctor_get(x_147, 0); +x_150 = lean_ctor_get(x_147, 1); +x_151 = lean_ctor_get(x_149, 0); +lean_inc(x_151); +lean_dec(x_149); +x_192 = l_Lean_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__2___closed__3; +lean_ctor_set(x_147, 1, x_151); +lean_ctor_set(x_147, 0, x_192); +x_193 = l_Lean_Expr_hasFVar(x_145); +if (x_193 == 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; -x_16 = lean_ctor_get(x_2, 1); -x_17 = lean_ctor_get(x_14, 1); -x_18 = lean_ctor_get(x_14, 2); -lean_inc(x_1); -x_19 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27(x_1, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_19, 1); -lean_inc(x_21); -lean_dec(x_19); -x_22 = lean_box(0); -lean_inc(x_1); -x_23 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam___spec__1(x_1, x_18, x_22, x_4, x_5, x_6, x_7, x_8, x_9, x_21); -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_23, 1); -lean_inc(x_25); -lean_dec(x_23); -lean_ctor_set(x_14, 2, x_24); -lean_ctor_set(x_14, 1, x_20); -lean_ctor_set(x_2, 1, x_3); +uint8_t x_194; +x_194 = l_Lean_Expr_hasMVar(x_145); +if (x_194 == 0) { -lean_object* _tmp_1 = x_16; -lean_object* _tmp_2 = x_2; -lean_object* _tmp_9 = x_25; -x_2 = _tmp_1; -x_3 = _tmp_2; -x_10 = _tmp_9; -} -goto _start; +uint8_t x_195; +lean_dec(x_145); +x_195 = 0; +x_178 = x_195; +x_179 = x_147; +goto block_191; } 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; -x_27 = lean_ctor_get(x_2, 1); -x_28 = lean_ctor_get(x_14, 0); -x_29 = lean_ctor_get(x_14, 1); -x_30 = lean_ctor_get(x_14, 2); -lean_inc(x_30); -lean_inc(x_29); -lean_inc(x_28); -lean_dec(x_14); -lean_inc(x_1); -x_31 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27(x_1, x_29, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -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_1); -x_35 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam___spec__1(x_1, x_30, x_34, x_4, x_5, x_6, x_7, x_8, x_9, x_33); -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(0, 3, 0); -lean_ctor_set(x_38, 0, x_28); -lean_ctor_set(x_38, 1, x_32); -lean_ctor_set(x_38, 2, x_36); -lean_ctor_set(x_2, 1, x_3); -lean_ctor_set(x_2, 0, x_38); -{ -lean_object* _tmp_1 = x_27; -lean_object* _tmp_2 = x_2; -lean_object* _tmp_9 = x_37; -x_2 = _tmp_1; -x_3 = _tmp_2; -x_10 = _tmp_9; -} -goto _start; +lean_object* x_196; lean_object* x_197; lean_object* x_198; uint8_t x_199; +lean_inc(x_3); +lean_inc(x_2); +x_196 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit(x_2, x_3, x_145, x_147); +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_unbox(x_197); +lean_dec(x_197); +x_178 = x_199; +x_179 = x_198; +goto block_191; } } 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; -x_40 = lean_ctor_get(x_2, 0); -x_41 = lean_ctor_get(x_2, 1); -lean_inc(x_41); -lean_inc(x_40); -lean_dec(x_2); -x_42 = lean_ctor_get(x_40, 0); -lean_inc(x_42); -x_43 = lean_ctor_get(x_40, 1); -lean_inc(x_43); -x_44 = lean_ctor_get(x_40, 2); -lean_inc(x_44); -if (lean_is_exclusive(x_40)) { - lean_ctor_release(x_40, 0); - lean_ctor_release(x_40, 1); - lean_ctor_release(x_40, 2); - x_45 = x_40; -} else { - lean_dec_ref(x_40); - x_45 = lean_box(0); -} -lean_inc(x_1); -x_46 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27(x_1, x_43, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -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_box(0); -lean_inc(x_1); -x_50 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam___spec__1(x_1, x_44, x_49, x_4, x_5, x_6, x_7, x_8, x_9, x_48); -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); -if (lean_is_scalar(x_45)) { - x_53 = lean_alloc_ctor(0, 3, 0); -} else { - x_53 = x_45; -} -lean_ctor_set(x_53, 0, x_42); -lean_ctor_set(x_53, 1, x_47); -lean_ctor_set(x_53, 2, x_51); -x_54 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_54, 0, x_53); -lean_ctor_set(x_54, 1, x_3); -x_2 = x_41; -x_3 = x_54; -x_10 = x_52; -goto _start; -} -} -} +lean_object* x_200; lean_object* x_201; lean_object* x_202; uint8_t x_203; +lean_inc(x_3); +lean_inc(x_2); +x_200 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit(x_2, x_3, x_145, x_147); +x_201 = lean_ctor_get(x_200, 0); +lean_inc(x_201); +x_202 = lean_ctor_get(x_200, 1); +lean_inc(x_202); +lean_dec(x_200); +x_203 = lean_unbox(x_201); +lean_dec(x_201); +x_178 = x_203; +x_179 = x_202; +goto block_191; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_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) { -_start: +block_177: { -lean_object* x_10; lean_object* x_11; -x_10 = lean_box(0); -x_11 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam___spec__2(x_2, x_1, x_10, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_11; -} +lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; uint8_t x_158; +x_154 = lean_ctor_get(x_153, 1); +lean_inc(x_154); +lean_dec(x_153); +x_155 = lean_st_ref_take(x_5, x_150); +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_is_exclusive(x_156); +if (x_158 == 0) +{ +lean_object* x_159; lean_object* x_160; uint8_t x_161; +x_159 = lean_ctor_get(x_156, 0); +lean_dec(x_159); +lean_ctor_set(x_156, 0, x_154); +x_160 = lean_st_ref_set(x_5, x_156, x_157); +x_161 = !lean_is_exclusive(x_160); +if (x_161 == 0) +{ +lean_object* x_162; lean_object* x_163; +x_162 = lean_ctor_get(x_160, 0); +lean_dec(x_162); +x_163 = lean_box(x_152); +lean_ctor_set(x_160, 0, x_163); +return x_160; } -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam___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: +else { -lean_object* x_11; -x_11 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam___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); -return x_11; +lean_object* x_164; lean_object* x_165; lean_object* x_166; +x_164 = lean_ctor_get(x_160, 1); +lean_inc(x_164); +lean_dec(x_160); +x_165 = lean_box(x_152); +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_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam___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: +else { -lean_object* x_11; -x_11 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam___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); -return x_11; +lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; +x_167 = lean_ctor_get(x_156, 1); +x_168 = lean_ctor_get(x_156, 2); +x_169 = lean_ctor_get(x_156, 3); +x_170 = lean_ctor_get(x_156, 4); +lean_inc(x_170); +lean_inc(x_169); +lean_inc(x_168); +lean_inc(x_167); +lean_dec(x_156); +x_171 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_171, 0, x_154); +lean_ctor_set(x_171, 1, x_167); +lean_ctor_set(x_171, 2, x_168); +lean_ctor_set(x_171, 3, x_169); +lean_ctor_set(x_171, 4, x_170); +x_172 = lean_st_ref_set(x_5, x_171, x_157); +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_172); + x_174 = lean_box(0); } +x_175 = lean_box(x_152); +if (lean_is_scalar(x_174)) { + x_176 = lean_alloc_ctor(0, 2, 0); +} else { + x_176 = x_174; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_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) { -_start: -{ -lean_object* x_10; -x_10 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -return x_10; +lean_ctor_set(x_176, 0, x_175); +lean_ctor_set(x_176, 1, x_173); +return x_176; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkResultUniverse(lean_object* x_1, lean_object* x_2, uint8_t x_3) { -_start: +block_191: { -uint8_t x_4; -x_4 = l_Array_isEmpty___rarg(x_1); -if (x_4 == 0) +if (x_178 == 0) { -lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; -x_5 = lean_array_to_list(x_1); -x_6 = l_Lean_Level_mkNaryMax(x_5); -x_7 = lean_unsigned_to_nat(0u); -x_8 = lean_nat_dec_eq(x_2, x_7); -if (x_8 == 0) +uint8_t x_180; +x_180 = l_Lean_Expr_hasFVar(x_146); +if (x_180 == 0) { -lean_object* x_9; -x_9 = l_Lean_Level_normalize(x_6); -lean_dec(x_6); -return x_9; +uint8_t x_181; +x_181 = l_Lean_Expr_hasMVar(x_146); +if (x_181 == 0) +{ +uint8_t x_182; +lean_dec(x_146); +lean_dec(x_3); +lean_dec(x_2); +x_182 = 0; +x_152 = x_182; +x_153 = x_179; +goto block_177; } else { -uint8_t x_10; -x_10 = l_Lean_Level_isZero(x_6); -if (x_10 == 0) -{ -uint8_t x_11; -x_11 = l_Lean_Level_isNeverZero(x_6); -if (x_11 == 0) -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_12 = l_Lean_levelOne; -x_13 = l_Lean_Level_max___override(x_6, x_12); -x_14 = l_Lean_Level_normalize(x_13); -lean_dec(x_13); -return x_14; +lean_object* x_183; lean_object* x_184; lean_object* x_185; uint8_t x_186; +x_183 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit(x_2, x_3, x_146, x_179); +x_184 = lean_ctor_get(x_183, 0); +lean_inc(x_184); +x_185 = lean_ctor_get(x_183, 1); +lean_inc(x_185); +lean_dec(x_183); +x_186 = lean_unbox(x_184); +lean_dec(x_184); +x_152 = x_186; +x_153 = x_185; +goto block_177; +} } else { -lean_object* x_15; -x_15 = l_Lean_Level_normalize(x_6); -lean_dec(x_6); -return x_15; +lean_object* x_187; lean_object* x_188; lean_object* x_189; uint8_t x_190; +x_187 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit(x_2, x_3, x_146, x_179); +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); +x_190 = lean_unbox(x_188); +lean_dec(x_188); +x_152 = x_190; +x_153 = x_189; +goto block_177; } } else { -lean_object* x_16; -x_16 = l_Lean_Level_normalize(x_6); -lean_dec(x_6); -return x_16; +lean_dec(x_146); +lean_dec(x_3); +lean_dec(x_2); +x_152 = x_178; +x_153 = x_179; +goto block_177; } } } else { -lean_object* x_17; uint8_t x_18; -x_17 = lean_unsigned_to_nat(0u); -x_18 = lean_nat_dec_eq(x_2, x_17); -if (x_18 == 0) +lean_object* x_204; lean_object* x_205; lean_object* x_206; uint8_t x_207; lean_object* x_208; uint8_t x_225; lean_object* x_226; lean_object* x_239; lean_object* x_240; uint8_t x_241; +x_204 = lean_ctor_get(x_147, 0); +x_205 = lean_ctor_get(x_147, 1); +lean_inc(x_205); +lean_inc(x_204); +lean_dec(x_147); +x_206 = lean_ctor_get(x_204, 0); +lean_inc(x_206); +lean_dec(x_204); +x_239 = l_Lean_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__2___closed__3; +x_240 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_240, 0, x_239); +lean_ctor_set(x_240, 1, x_206); +x_241 = l_Lean_Expr_hasFVar(x_145); +if (x_241 == 0) { -lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_19 = lean_array_to_list(x_1); -x_20 = l_Lean_Level_mkNaryMax(x_19); -x_21 = l_Lean_Level_normalize(x_20); -lean_dec(x_20); -return x_21; +uint8_t x_242; +x_242 = l_Lean_Expr_hasMVar(x_145); +if (x_242 == 0) +{ +uint8_t x_243; +lean_dec(x_145); +x_243 = 0; +x_225 = x_243; +x_226 = x_240; +goto block_238; } else { -lean_dec(x_1); -if (x_3 == 0) -{ -lean_object* x_22; -x_22 = l_Lean_levelOne; -return x_22; +lean_object* x_244; lean_object* x_245; lean_object* x_246; uint8_t x_247; +lean_inc(x_3); +lean_inc(x_2); +x_244 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit(x_2, x_3, x_145, x_240); +x_245 = lean_ctor_get(x_244, 0); +lean_inc(x_245); +x_246 = lean_ctor_get(x_244, 1); +lean_inc(x_246); +lean_dec(x_244); +x_247 = lean_unbox(x_245); +lean_dec(x_245); +x_225 = x_247; +x_226 = x_246; +goto block_238; +} } else { -lean_object* x_23; -x_23 = l_Lean_levelZero; -return x_23; -} +lean_object* x_248; lean_object* x_249; lean_object* x_250; uint8_t x_251; +lean_inc(x_3); +lean_inc(x_2); +x_248 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit(x_2, x_3, x_145, x_240); +x_249 = lean_ctor_get(x_248, 0); +lean_inc(x_249); +x_250 = lean_ctor_get(x_248, 1); +lean_inc(x_250); +lean_dec(x_248); +x_251 = lean_unbox(x_249); +lean_dec(x_249); +x_225 = x_251; +x_226 = x_250; +goto block_238; } +block_224: +{ +lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; +x_209 = lean_ctor_get(x_208, 1); +lean_inc(x_209); +lean_dec(x_208); +x_210 = lean_st_ref_take(x_5, x_205); +x_211 = lean_ctor_get(x_210, 0); +lean_inc(x_211); +x_212 = lean_ctor_get(x_210, 1); +lean_inc(x_212); +lean_dec(x_210); +x_213 = lean_ctor_get(x_211, 1); +lean_inc(x_213); +x_214 = lean_ctor_get(x_211, 2); +lean_inc(x_214); +x_215 = lean_ctor_get(x_211, 3); +lean_inc(x_215); +x_216 = lean_ctor_get(x_211, 4); +lean_inc(x_216); +if (lean_is_exclusive(x_211)) { + lean_ctor_release(x_211, 0); + lean_ctor_release(x_211, 1); + lean_ctor_release(x_211, 2); + lean_ctor_release(x_211, 3); + lean_ctor_release(x_211, 4); + x_217 = x_211; +} else { + lean_dec_ref(x_211); + x_217 = lean_box(0); } +if (lean_is_scalar(x_217)) { + x_218 = lean_alloc_ctor(0, 5, 0); +} else { + x_218 = x_217; } +lean_ctor_set(x_218, 0, x_209); +lean_ctor_set(x_218, 1, x_213); +lean_ctor_set(x_218, 2, x_214); +lean_ctor_set(x_218, 3, x_215); +lean_ctor_set(x_218, 4, x_216); +x_219 = lean_st_ref_set(x_5, x_218, x_212); +x_220 = lean_ctor_get(x_219, 1); +lean_inc(x_220); +if (lean_is_exclusive(x_219)) { + lean_ctor_release(x_219, 0); + lean_ctor_release(x_219, 1); + x_221 = x_219; +} else { + lean_dec_ref(x_219); + x_221 = lean_box(0); } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkResultUniverse___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_Elab_Command_mkResultUniverse(x_1, x_2, x_4); -lean_dec(x_2); -return x_5; +x_222 = lean_box(x_207); +if (lean_is_scalar(x_221)) { + x_223 = lean_alloc_ctor(0, 2, 0); +} else { + x_223 = x_221; } +lean_ctor_set(x_223, 0, x_222); +lean_ctor_set(x_223, 1, x_220); +return x_223; } -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Command_accLevel_go___spec__2(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4) { -_start: +block_238: { -uint8_t x_5; -x_5 = lean_usize_dec_eq(x_3, x_4); -if (x_5 == 0) +if (x_225 == 0) { -lean_object* x_6; uint8_t x_7; -x_6 = lean_array_uget(x_2, x_3); -x_7 = lean_level_eq(x_6, x_1); -lean_dec(x_6); -if (x_7 == 0) +uint8_t x_227; +x_227 = l_Lean_Expr_hasFVar(x_146); +if (x_227 == 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_228; +x_228 = l_Lean_Expr_hasMVar(x_146); +if (x_228 == 0) { -uint8_t x_11; -x_11 = 1; -return x_11; +uint8_t x_229; +lean_dec(x_146); +lean_dec(x_3); +lean_dec(x_2); +x_229 = 0; +x_207 = x_229; +x_208 = x_226; +goto block_224; +} +else +{ +lean_object* x_230; lean_object* x_231; lean_object* x_232; uint8_t x_233; +x_230 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit(x_2, x_3, x_146, x_226); +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); +x_233 = lean_unbox(x_231); +lean_dec(x_231); +x_207 = x_233; +x_208 = x_232; +goto block_224; } } else { -uint8_t x_12; -x_12 = 0; -return x_12; +lean_object* x_234; lean_object* x_235; lean_object* x_236; uint8_t x_237; +x_234 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit(x_2, x_3, x_146, x_226); +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_unbox(x_235); +lean_dec(x_235); +x_207 = x_237; +x_208 = x_236; +goto block_224; +} +} +else +{ +lean_dec(x_146); +lean_dec(x_3); +lean_dec(x_2); +x_207 = x_225; +x_208 = x_226; +goto block_224; } } } -LEAN_EXPORT uint8_t l_Array_contains___at_Lean_Elab_Command_accLevel_go___spec__1(lean_object* x_1, lean_object* x_2) { +} +} +} +LEAN_EXPORT lean_object* l_Array_erase___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__3(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; +x_3 = lean_unsigned_to_nat(0u); +x_4 = l_Array_indexOfAux___at___private_Lean_Meta_Constructions_BRecOn_0__Lean_buildBRecOnMinorPremise_go___spec__1(x_1, x_2, x_3); +if (lean_obj_tag(x_4) == 0) +{ +return x_1; +} +else +{ +lean_object* x_5; lean_object* x_6; +x_5 = lean_ctor_get(x_4, 0); +lean_inc(x_5); +lean_dec(x_4); +x_6 = l_Array_feraseIdx___rarg(x_1, x_5); +return x_6; +} +} +} +LEAN_EXPORT uint8_t l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__1(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; lean_object* x_4; uint8_t x_5; @@ -11477,1692 +12652,1198 @@ size_t x_7; size_t x_8; uint8_t x_9; x_7 = 0; x_8 = lean_usize_of_nat(x_3); lean_dec(x_3); -x_9 = l_Array_anyMUnsafe_any___at_Lean_Elab_Command_accLevel_go___spec__2(x_2, x_1, x_7, x_8); +x_9 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__1(x_2, x_1, x_7, x_8); return x_9; } } } -static lean_object* _init_l_Lean_Elab_Command_accLevel_go___closed__1() { +LEAN_EXPORT uint8_t l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__2(lean_object* x_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); +uint8_t x_2; +x_2 = 0; return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_accLevel_go(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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___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_5; -switch (lean_obj_tag(x_2)) { -case 0: +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +lean_inc(x_1); +x_10 = lean_array_push(x_3, x_1); +x_11 = l_Array_erase___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__3(x_2, x_1); +lean_dec(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_10); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_12); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_13); +lean_ctor_set(x_14, 1, x_9); +return x_14; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__4___closed__1() { +_start: { -lean_object* x_20; lean_object* x_21; -lean_dec(x_3); -x_20 = l_Lean_Elab_Command_accLevel_go___closed__1; -x_21 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_21, 0, x_20); -lean_ctor_set(x_21, 1, x_4); -return x_21; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__2___boxed), 1, 0); +return x_1; } -case 1: +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___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_22; lean_object* x_23; uint8_t x_24; -x_22 = lean_ctor_get(x_2, 0); -lean_inc(x_22); -x_23 = lean_unsigned_to_nat(0u); -x_24 = lean_nat_dec_eq(x_3, x_23); -if (x_24 == 0) +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +lean_inc(x_3); +x_11 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__1___boxed), 2, 1); +lean_closure_set(x_11, 0, x_3); +x_12 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__4___closed__1; +x_13 = l_Lean_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__2(x_1, x_11, x_12, x_6, x_7, x_8, x_9, x_10); +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_unbox(x_14); +lean_dec(x_14); +if (x_15 == 0) { -lean_object* x_25; lean_object* x_26; -lean_dec(x_2); -x_25 = lean_unsigned_to_nat(1u); -x_26 = lean_nat_sub(x_3, x_25); -lean_dec(x_3); -x_2 = x_22; -x_3 = x_26; -goto _start; +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_13, 1); +lean_inc(x_16); +lean_dec(x_13); +x_17 = lean_box(0); +x_18 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__3(x_2, x_3, x_4, x_17, x_6, x_7, x_8, x_9, x_16); +return x_18; } else { -uint8_t x_28; -lean_dec(x_22); -lean_dec(x_3); -x_28 = lean_level_eq(x_2, x_1); -if (x_28 == 0) -{ -uint8_t x_29; -x_29 = l_Lean_Level_occurs(x_1, x_2); -if (x_29 == 0) -{ -uint8_t x_30; -x_30 = l_Array_contains___at_Lean_Elab_Command_accLevel_go___spec__1(x_4, x_2); -if (x_30 == 0) +uint8_t x_19; +lean_dec(x_2); +x_19 = !lean_is_exclusive(x_13); +if (x_19 == 0) { -lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_31 = lean_array_push(x_4, x_2); -x_32 = l_Lean_Elab_Command_accLevel_go___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); -return x_33; +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_13, 0); +lean_dec(x_20); +x_21 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_21, 0, x_3); +lean_ctor_set(x_21, 1, x_4); +x_22 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_22, 0, x_21); +lean_ctor_set(x_13, 0, x_22); +return x_13; } else { -lean_object* x_34; lean_object* x_35; -lean_dec(x_2); -x_34 = l_Lean_Elab_Command_accLevel_go___closed__1; -x_35 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_35, 0, x_34); -lean_ctor_set(x_35, 1, x_4); -return x_35; +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_23 = lean_ctor_get(x_13, 1); +lean_inc(x_23); +lean_dec(x_13); +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_3); +lean_ctor_set(x_24, 1, x_4); +x_25 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_25, 0, x_24); +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_23); +return x_26; } } -else +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___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) { +_start: { -lean_object* x_36; lean_object* x_37; +lean_object* x_11; uint8_t x_12; +x_11 = l_Lean_LocalDecl_userName(x_1); +x_12 = l_Lean_Name_hasMacroScopes(x_11); +lean_dec(x_11); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_dec(x_2); -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_4); -return x_37; -} +lean_dec(x_1); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_3); +lean_ctor_set(x_13, 1, x_4); +x_14 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_14, 0, x_13); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_10); +return x_15; } else { -lean_object* x_38; lean_object* x_39; -lean_dec(x_2); -x_38 = l_Lean_Elab_Command_accLevel_go___closed__1; -x_39 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_39, 0, x_38); -lean_ctor_set(x_39, 1, x_4); -return x_39; +lean_object* x_16; lean_object* x_17; +x_16 = lean_box(0); +x_17 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__4(x_1, x_2, x_3, x_4, x_16, x_6, x_7, x_8, x_9, x_10); +return x_17; } } } -case 4: +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: { -lean_object* x_40; uint8_t x_41; -x_40 = lean_unsigned_to_nat(0u); -x_41 = lean_nat_dec_eq(x_3, x_40); -if (x_41 == 0) +lean_object* x_10; +lean_inc(x_5); +x_10 = l_Lean_Meta_getFVarLocalDecl(x_1, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_10) == 0) { -lean_object* x_42; -x_42 = lean_box(0); -x_5 = x_42; -goto block_19; -} -else +uint8_t x_11; +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) { -uint8_t x_43; -x_43 = lean_level_eq(x_2, x_1); -if (x_43 == 0) +lean_object* x_12; lean_object* x_13; uint8_t x_14; uint8_t x_15; +x_12 = lean_ctor_get(x_10, 0); +x_13 = lean_ctor_get(x_10, 1); +x_14 = l_Lean_LocalDecl_binderInfo(x_12); +x_15 = l_Lean_BinderInfo_isExplicit(x_14); +if (x_15 == 0) { -lean_object* x_44; -x_44 = lean_box(0); -x_5 = x_44; -goto block_19; +lean_object* x_16; lean_object* x_17; +lean_free_object(x_10); +x_16 = lean_box(0); +x_17 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__5(x_12, x_1, x_2, x_3, x_16, x_5, x_6, x_7, x_8, x_13); +lean_dec(x_5); +return x_17; } else { -lean_object* x_45; lean_object* x_46; -lean_dec(x_3); -lean_dec(x_2); -x_45 = l_Lean_Elab_Command_accLevel_go___closed__1; -x_46 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_46, 0, x_45); -lean_ctor_set(x_46, 1, x_4); -return x_46; -} -} +lean_object* x_18; lean_object* x_19; +lean_dec(x_12); +lean_dec(x_5); +lean_dec(x_1); +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_2); +lean_ctor_set(x_18, 1, x_3); +x_19 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set(x_10, 0, x_19); +return x_10; } -case 5: -{ -lean_object* x_47; uint8_t x_48; -x_47 = lean_unsigned_to_nat(0u); -x_48 = lean_nat_dec_eq(x_3, x_47); -if (x_48 == 0) -{ -lean_object* x_49; -x_49 = lean_box(0); -x_5 = x_49; -goto block_19; } else { -uint8_t x_50; -x_50 = lean_level_eq(x_2, x_1); -if (x_50 == 0) +lean_object* x_20; lean_object* x_21; uint8_t x_22; uint8_t x_23; +x_20 = lean_ctor_get(x_10, 0); +x_21 = lean_ctor_get(x_10, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_10); +x_22 = l_Lean_LocalDecl_binderInfo(x_20); +x_23 = l_Lean_BinderInfo_isExplicit(x_22); +if (x_23 == 0) { -lean_object* x_51; -x_51 = lean_box(0); -x_5 = x_51; -goto block_19; +lean_object* x_24; lean_object* x_25; +x_24 = lean_box(0); +x_25 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__5(x_20, x_1, x_2, x_3, x_24, x_5, x_6, x_7, x_8, x_21); +lean_dec(x_5); +return x_25; } else { -lean_object* x_52; lean_object* x_53; -lean_dec(x_3); -lean_dec(x_2); -x_52 = l_Lean_Elab_Command_accLevel_go___closed__1; -x_53 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_53, 0, x_52); -lean_ctor_set(x_53, 1, x_4); -return x_53; +lean_object* x_26; lean_object* x_27; lean_object* x_28; +lean_dec(x_20); +lean_dec(x_5); +lean_dec(x_1); +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_2); +lean_ctor_set(x_26, 1, x_3); +x_27 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_27, 0, 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_21); +return x_28; } } } -default: -{ -lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; -x_54 = lean_ctor_get(x_2, 0); -lean_inc(x_54); -x_55 = lean_ctor_get(x_2, 1); -lean_inc(x_55); -lean_dec(x_2); -lean_inc(x_3); -x_56 = l_Lean_Elab_Command_accLevel_go(x_1, x_54, x_3, x_4); -x_57 = lean_ctor_get(x_56, 0); -lean_inc(x_57); -if (lean_obj_tag(x_57) == 0) +else { -uint8_t x_58; -lean_dec(x_55); +uint8_t x_29; +lean_dec(x_5); lean_dec(x_3); -x_58 = !lean_is_exclusive(x_56); -if (x_58 == 0) +lean_dec(x_2); +lean_dec(x_1); +x_29 = !lean_is_exclusive(x_10); +if (x_29 == 0) { -lean_object* x_59; lean_object* x_60; -x_59 = lean_ctor_get(x_56, 0); -lean_dec(x_59); -x_60 = lean_box(0); -lean_ctor_set(x_56, 0, x_60); -return x_56; +return x_10; } else { -lean_object* x_61; lean_object* x_62; lean_object* x_63; -x_61 = lean_ctor_get(x_56, 1); -lean_inc(x_61); -lean_dec(x_56); -x_62 = lean_box(0); -x_63 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_63, 0, x_62); -lean_ctor_set(x_63, 1, x_61); -return x_63; -} +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_dec(x_10); +x_32 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_31); +return x_32; } -else -{ -lean_object* x_64; -lean_dec(x_57); -x_64 = lean_ctor_get(x_56, 1); -lean_inc(x_64); -lean_dec(x_56); -x_2 = x_55; -x_4 = x_64; -goto _start; } } } -block_19: +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___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) { +_start: { -uint8_t x_6; +uint8_t x_10; +x_10 = lean_usize_dec_lt(x_3, x_2); +if (x_10 == 0) +{ +lean_object* x_11; lean_dec(x_5); -x_6 = l_Lean_Level_occurs(x_1, x_2); -if (x_6 == 0) +x_11 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_11, 0, x_4); +lean_ctor_set(x_11, 1, x_9); +return x_11; +} +else { -lean_object* x_7; uint8_t x_8; -x_7 = lean_unsigned_to_nat(0u); -x_8 = lean_nat_dec_lt(x_7, x_3); -lean_dec(x_3); -if (x_8 == 0) +lean_object* x_12; uint8_t x_13; +x_12 = lean_array_uget(x_1, x_3); +x_13 = !lean_is_exclusive(x_4); +if (x_13 == 0) { -uint8_t x_9; -x_9 = l_Array_contains___at_Lean_Elab_Command_accLevel_go___spec__1(x_4, x_2); -if (x_9 == 0) +lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_14 = lean_ctor_get(x_4, 0); +x_15 = lean_ctor_get(x_4, 1); +x_16 = l_Lean_Expr_isFVar(x_12); +if (x_16 == 0) { -lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_10 = lean_array_push(x_4, x_2); -x_11 = l_Lean_Elab_Command_accLevel_go___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); -return x_12; +lean_object* x_17; +lean_dec(x_12); +lean_dec(x_5); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_4); +lean_ctor_set(x_17, 1, x_9); +return x_17; } else { -lean_object* x_13; lean_object* x_14; -lean_dec(x_2); -x_13 = l_Lean_Elab_Command_accLevel_go___closed__1; -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_13); -lean_ctor_set(x_14, 1, x_4); -return x_14; -} -} -else +uint8_t x_18; +x_18 = l_Array_contains___at_Lean_Meta_setMVarUserNamesAt___spec__1(x_14, x_12); +if (x_18 == 0) { -lean_object* x_15; lean_object* x_16; -lean_dec(x_2); -x_15 = lean_box(0); -x_16 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_16, 0, x_15); -lean_ctor_set(x_16, 1, x_4); -return x_16; -} +lean_object* x_19; +lean_dec(x_12); +lean_dec(x_5); +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_4); +lean_ctor_set(x_19, 1, x_9); +return x_19; } else { -lean_object* x_17; lean_object* x_18; -lean_dec(x_3); -lean_dec(x_2); -x_17 = lean_box(0); -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_17); -lean_ctor_set(x_18, 1, x_4); -return x_18; -} -} -} -} -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Command_accLevel_go___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_Command_accLevel_go___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_Command_accLevel_go___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_Command_accLevel_go___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_Lean_Elab_Command_accLevel_go___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -lean_object* x_5; -x_5 = l_Lean_Elab_Command_accLevel_go(x_1, x_2, x_3, x_4); -lean_dec(x_1); -return x_5; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Command_accLevel(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -lean_object* x_5; -x_5 = l_Lean_Elab_Command_accLevel_go(x_2, x_1, x_3, x_4); -return x_5; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Command_accLevel___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -lean_object* x_5; -x_5 = l_Lean_Elab_Command_accLevel(x_1, x_2, x_3, x_4); -lean_dec(x_2); -return x_5; -} -} -LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_accLevelAtCtor___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +lean_object* x_20; lean_object* x_21; +lean_free_object(x_4); +x_20 = lean_box(0); +lean_inc(x_5); +x_21 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__6(x_12, x_14, x_15, x_20, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_21) == 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_st_ref_get(x_6, 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, 0); -lean_inc(x_13); -lean_dec(x_11); -x_14 = lean_instantiate_level_mvars(x_13, x_1); -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_take(x_6, x_12); -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_17, 1); -lean_inc(x_19); -lean_dec(x_17); -x_20 = !lean_is_exclusive(x_18); -if (x_20 == 0) +lean_object* x_22; +x_22 = lean_ctor_get(x_21, 0); +lean_inc(x_22); +if (lean_obj_tag(x_22) == 0) { -lean_object* x_21; lean_object* x_22; uint8_t x_23; -x_21 = lean_ctor_get(x_18, 0); -lean_dec(x_21); -lean_ctor_set(x_18, 0, x_15); -x_22 = lean_st_ref_set(x_6, x_18, x_19); -x_23 = !lean_is_exclusive(x_22); +uint8_t x_23; +lean_dec(x_5); +x_23 = !lean_is_exclusive(x_21); if (x_23 == 0) { -lean_object* x_24; -x_24 = lean_ctor_get(x_22, 0); +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_21, 0); lean_dec(x_24); -lean_ctor_set(x_22, 0, x_16); -return x_22; +x_25 = lean_ctor_get(x_22, 0); +lean_inc(x_25); +lean_dec(x_22); +lean_ctor_set(x_21, 0, x_25); +return x_21; } else { -lean_object* x_25; lean_object* x_26; -x_25 = lean_ctor_get(x_22, 1); -lean_inc(x_25); +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_21, 1); +lean_inc(x_26); +lean_dec(x_21); +x_27 = lean_ctor_get(x_22, 0); +lean_inc(x_27); lean_dec(x_22); -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_16); -lean_ctor_set(x_26, 1, x_25); -return 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_26); +return x_28; } } 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; -x_27 = lean_ctor_get(x_18, 1); -x_28 = lean_ctor_get(x_18, 2); -x_29 = lean_ctor_get(x_18, 3); -x_30 = lean_ctor_get(x_18, 4); -lean_inc(x_30); +lean_object* x_29; lean_object* x_30; size_t x_31; size_t x_32; +x_29 = lean_ctor_get(x_21, 1); lean_inc(x_29); -lean_inc(x_28); -lean_inc(x_27); -lean_dec(x_18); -x_31 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_31, 0, x_15); -lean_ctor_set(x_31, 1, x_27); -lean_ctor_set(x_31, 2, x_28); -lean_ctor_set(x_31, 3, x_29); -lean_ctor_set(x_31, 4, x_30); -x_32 = lean_st_ref_set(x_6, x_31, x_19); -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); -} -if (lean_is_scalar(x_34)) { - x_35 = lean_alloc_ctor(0, 2, 0); -} else { - x_35 = x_34; -} -lean_ctor_set(x_35, 0, x_16); -lean_ctor_set(x_35, 1, x_33); -return x_35; -} +lean_dec(x_21); +x_30 = lean_ctor_get(x_22, 0); +lean_inc(x_30); +lean_dec(x_22); +x_31 = 1; +x_32 = lean_usize_add(x_3, x_31); +x_3 = x_32; +x_4 = x_30; +x_9 = x_29; +goto _start; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_accLevelAtCtor___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +else { -lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_10 = lean_ctor_get(x_7, 5); -x_11 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_1, x_5, x_6, x_7, x_8, x_9); -x_12 = !lean_is_exclusive(x_11); -if (x_12 == 0) +uint8_t x_34; +lean_dec(x_5); +x_34 = !lean_is_exclusive(x_21); +if (x_34 == 0) { -lean_object* x_13; lean_object* x_14; -x_13 = lean_ctor_get(x_11, 0); -lean_inc(x_10); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_10); -lean_ctor_set(x_14, 1, x_13); -lean_ctor_set_tag(x_11, 1); -lean_ctor_set(x_11, 0, x_14); -return x_11; +return x_21; } 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); -lean_inc(x_10); -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_10); -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_16); -return x_18; -} -} +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_21, 0); +x_36 = lean_ctor_get(x_21, 1); +lean_inc(x_36); +lean_inc(x_35); +lean_dec(x_21); +x_37 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +return x_37; } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_accLevelAtCtor___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; -x_11 = l_Lean_throwError___at_Lean_Elab_Command_accLevelAtCtor___spec__2(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_11; } } -static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked(" has type", 9, 9); -return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__2() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__3() { -_start: +lean_object* x_38; lean_object* x_39; uint8_t x_40; +x_38 = lean_ctor_get(x_4, 0); +x_39 = lean_ctor_get(x_4, 1); +lean_inc(x_39); +lean_inc(x_38); +lean_dec(x_4); +x_40 = l_Lean_Expr_isFVar(x_12); +if (x_40 == 0) { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("\ninductive type resulting type", 30, 30); -return x_1; -} +lean_object* x_41; lean_object* x_42; +lean_dec(x_12); +lean_dec(x_5); +x_41 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_41, 0, x_38); +lean_ctor_set(x_41, 1, x_39); +x_42 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_42, 0, x_41); +lean_ctor_set(x_42, 1, x_9); +return x_42; } -static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__4() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__3; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__5() { -_start: +uint8_t x_43; +x_43 = l_Array_contains___at_Lean_Meta_setMVarUserNamesAt___spec__1(x_38, x_12); +if (x_43 == 0) { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Command_accLevelAtCtor___lambda__1___boxed), 10, 0); -return x_1; -} +lean_object* x_44; lean_object* x_45; +lean_dec(x_12); +lean_dec(x_5); +x_44 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_44, 0, x_38); +lean_ctor_set(x_44, 1, x_39); +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; } -static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__6() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("\nrecall that Lean only infers the resulting universe level automatically when there is a unique solution for the universe level constraints, consider explicitly providing the inductive type resulting universe level", 214, 214); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__7() { -_start: +lean_object* x_46; lean_object* x_47; +x_46 = lean_box(0); +lean_inc(x_5); +x_47 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__6(x_12, x_38, x_39, x_46, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_47) == 0) { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__6; -x_2 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__8() { -_start: +lean_object* x_48; +x_48 = lean_ctor_get(x_47, 0); +lean_inc(x_48); +if (lean_obj_tag(x_48) == 0) { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__7; -x_2 = l_Lean_MessageData_ofFormat(x_1); -return x_2; +lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +lean_dec(x_5); +x_49 = lean_ctor_get(x_47, 1); +lean_inc(x_49); +if (lean_is_exclusive(x_47)) { + lean_ctor_release(x_47, 0); + lean_ctor_release(x_47, 1); + x_50 = x_47; +} else { + lean_dec_ref(x_47); + x_50 = lean_box(0); } +x_51 = lean_ctor_get(x_48, 0); +lean_inc(x_51); +lean_dec(x_48); +if (lean_is_scalar(x_50)) { + x_52 = lean_alloc_ctor(0, 2, 0); +} else { + x_52 = x_50; } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_accLevelAtCtor___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { -_start: -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; 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_15 = l_Lean_MessageData_ofExpr(x_1); -x_16 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5; -x_17 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_17, 0, x_16); -lean_ctor_set(x_17, 1, x_15); -x_18 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__6; -x_19 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_19, 0, x_17); -lean_ctor_set(x_19, 1, x_18); -x_20 = l_Lean_MessageData_ofExpr(x_2); -x_21 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_21, 0, x_19); -lean_ctor_set(x_21, 1, x_20); -x_22 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_22, 0, x_21); -lean_ctor_set(x_22, 1, x_16); -x_23 = l_Lean_indentD(x_22); -x_24 = l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__2; -x_25 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_25, 0, x_24); -lean_ctor_set(x_25, 1, x_23); -x_26 = l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__4; -x_27 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_26); -lean_inc(x_4); -x_28 = l_Lean_Level_addOffsetAux(x_3, x_4); -x_29 = l_Lean_Expr_sort___override(x_28); -x_30 = l_Lean_indentExpr(x_29); -x_31 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_31, 0, x_27); -lean_ctor_set(x_31, 1, x_30); -x_32 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_32, 0, x_31); -lean_ctor_set(x_32, 1, x_16); -x_33 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_33, 0, x_5); -lean_ctor_set(x_33, 1, x_32); -x_34 = l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__5; -x_35 = l_Lean_Level_isMVar(x_4); -lean_dec(x_4); -if (x_35 == 0) -{ -lean_object* x_36; lean_object* x_37; -x_36 = lean_box(0); -x_37 = lean_apply_10(x_34, x_33, x_36, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -return x_37; +lean_ctor_set(x_52, 0, x_51); +lean_ctor_set(x_52, 1, x_49); +return x_52; } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_38 = l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__8; -x_39 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_39, 0, x_33); -lean_ctor_set(x_39, 1, x_38); -x_40 = lean_box(0); -x_41 = lean_apply_10(x_34, x_39, x_40, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -return x_41; -} +lean_object* x_53; lean_object* x_54; size_t x_55; size_t x_56; +x_53 = lean_ctor_get(x_47, 1); +lean_inc(x_53); +lean_dec(x_47); +x_54 = lean_ctor_get(x_48, 0); +lean_inc(x_54); +lean_dec(x_48); +x_55 = 1; +x_56 = lean_usize_add(x_3, x_55); +x_3 = x_56; +x_4 = x_54; +x_9 = x_53; +goto _start; } } -static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("failed to compute resulting universe level of inductive datatype, constructor '", 79, 79); -return x_1; -} +lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; +lean_dec(x_5); +x_58 = lean_ctor_get(x_47, 0); +lean_inc(x_58); +x_59 = lean_ctor_get(x_47, 1); +lean_inc(x_59); +if (lean_is_exclusive(x_47)) { + lean_ctor_release(x_47, 0); + lean_ctor_release(x_47, 1); + x_60 = x_47; +} else { + lean_dec_ref(x_47); + x_60 = lean_box(0); } -static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_accLevelAtCtor___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +if (lean_is_scalar(x_60)) { + x_61 = lean_alloc_ctor(1, 2, 0); +} else { + x_61 = x_60; } +lean_ctor_set(x_61, 0, x_58); +lean_ctor_set(x_61, 1, x_59); +return x_61; } -static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("' has type", 10, 10); -return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_accLevelAtCtor___closed__3; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; } } -static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___closed__5() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("\nparameter", 10, 10); -return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___closed__6() { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___lambda__1___closed__1() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_accLevelAtCtor___closed__5; -x_2 = l_Lean_stringToMessageData(x_1); +x_1 = l_Lean_levelZero; +x_2 = l_Lean_Expr_sort___override(x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___closed__7() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___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; -x_1 = lean_mk_string_unchecked(" '", 2, 2); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___closed__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; size_t x_18; size_t x_19; lean_object* x_20; +x_9 = lean_unsigned_to_nat(0u); +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); +x_13 = lean_unsigned_to_nat(1u); +x_14 = lean_nat_sub(x_10, x_13); +lean_dec(x_10); +lean_inc(x_3); +x_15 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_3, x_12, x_14); +x_16 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__8___closed__1; +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_2); +lean_ctor_set(x_17, 1, x_16); +x_18 = lean_array_size(x_15); +x_19 = 0; +lean_inc(x_4); +x_20 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4(x_15, x_18, x_19, x_17, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_15); +if (lean_obj_tag(x_20) == 0) { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_accLevelAtCtor___closed__7; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___closed__9() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("'", 1, 1); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___closed__10() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_accLevelAtCtor___closed__9; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Command_accLevelAtCtor(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, 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_2); -x_13 = lean_infer_type(x_2, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_13) == 0) -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_14 = lean_ctor_get(x_13, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_13, 1); -lean_inc(x_15); -lean_dec(x_13); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_14); -x_16 = l_Lean_Meta_getLevel(x_14, x_8, x_9, x_10, x_11, x_15); -if (lean_obj_tag(x_16) == 0) -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_16, 1); -lean_inc(x_18); -lean_dec(x_16); -x_19 = l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_accLevelAtCtor___spec__1(x_17, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_18); -x_20 = !lean_is_exclusive(x_19); -if (x_20 == 0) -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; -x_21 = lean_ctor_get(x_19, 0); -x_22 = lean_ctor_get(x_19, 1); -x_23 = lean_st_ref_take(x_5, x_22); -x_24 = !lean_is_exclusive(x_23); -if (x_24 == 0) +uint8_t x_21; +x_21 = !lean_is_exclusive(x_20); +if (x_21 == 0) { -lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; -x_25 = lean_ctor_get(x_23, 0); -x_26 = lean_ctor_get(x_23, 1); -lean_inc(x_4); -x_27 = l_Lean_Elab_Command_accLevel_go(x_3, x_21, x_4, x_25); -x_28 = !lean_is_exclusive(x_27); -if (x_28 == 0) +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; +x_22 = lean_ctor_get(x_20, 0); +x_23 = lean_ctor_get(x_20, 1); +x_24 = lean_ctor_get(x_22, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_22, 1); +lean_inc(x_25); +lean_dec(x_22); +x_26 = l_Array_isEmpty___rarg(x_25); +if (x_26 == 0) { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_27, 0); -x_30 = lean_ctor_get(x_27, 1); -x_31 = lean_st_ref_set(x_5, x_30, x_26); -if (lean_obj_tag(x_29) == 0) +lean_object* x_27; uint8_t x_28; uint8_t x_29; uint8_t x_30; lean_object* x_31; +lean_free_object(x_20); +lean_dec(x_1); +lean_inc(x_25); +x_27 = l_Array_append___rarg(x_25, x_24); +lean_dec(x_24); +x_28 = 0; +x_29 = 1; +x_30 = 1; +lean_inc(x_3); +x_31 = l_Lean_Meta_mkForallFVars(x_27, x_3, x_28, x_29, x_30, x_4, x_5, x_6, x_7, x_23); +if (lean_obj_tag(x_31) == 0) { -lean_object* x_32; lean_object* x_33; -x_32 = lean_ctor_get(x_31, 1); +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); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_14); -x_33 = lean_infer_type(x_14, x_8, x_9, x_10, x_11, x_32); -if (lean_obj_tag(x_33) == 0) +x_34 = l_Lean_Expr_getAppFn(x_3); +lean_dec(x_3); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_35 = lean_infer_type(x_34, x_4, x_5, x_6, x_7, x_33); +if (lean_obj_tag(x_35) == 0) { -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_34 = lean_ctor_get(x_33, 0); -lean_inc(x_34); -x_35 = lean_ctor_get(x_33, 1); -lean_inc(x_35); -lean_dec(x_33); -x_36 = lean_ctor_get(x_1, 0); +lean_object* x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; +x_36 = lean_ctor_get(x_35, 0); lean_inc(x_36); -x_37 = l_Lean_MessageData_ofName(x_36); -x_38 = l_Lean_Elab_Command_accLevelAtCtor___closed__2; -lean_ctor_set_tag(x_27, 7); -lean_ctor_set(x_27, 1, x_37); -lean_ctor_set(x_27, 0, x_38); -x_39 = l_Lean_Elab_Command_accLevelAtCtor___closed__4; -lean_ctor_set_tag(x_23, 7); -lean_ctor_set(x_23, 1, x_39); -lean_ctor_set(x_23, 0, x_27); -x_40 = lean_ctor_get(x_1, 1); -lean_inc(x_40); -lean_dec(x_1); -x_41 = l_Lean_indentExpr(x_40); -lean_ctor_set_tag(x_19, 7); -lean_ctor_set(x_19, 1, x_41); -lean_ctor_set(x_19, 0, x_23); -x_42 = l_Lean_Elab_Command_accLevelAtCtor___closed__6; -x_43 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_43, 0, x_19); -lean_ctor_set(x_43, 1, x_42); -lean_inc(x_8); -x_44 = l_Lean_Meta_getFVarLocalDecl(x_2, x_8, x_9, x_10, x_11, x_35); -if (lean_obj_tag(x_44) == 0) +x_37 = lean_ctor_get(x_35, 1); +lean_inc(x_37); +lean_dec(x_35); +x_38 = l_Lean_instantiateMVars___at___private_Lean_Meta_Basic_0__Lean_Meta_isClassApp_x3f___spec__1(x_36, x_4, x_5, x_6, x_7, x_37); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_39 = !lean_is_exclusive(x_38); +if (x_39 == 0) { -lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; -x_45 = lean_ctor_get(x_44, 0); -lean_inc(x_45); -x_46 = lean_ctor_get(x_44, 1); -lean_inc(x_46); +lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_40 = lean_ctor_get(x_38, 0); +x_41 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getArrowBinderNames(x_40); +x_42 = lean_array_get_size(x_25); +lean_dec(x_25); +x_43 = l_Array_toSubarray___rarg(x_41, x_9, x_42); +x_44 = l_Array_ofSubarray___rarg(x_43); +lean_dec(x_43); +x_45 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceArrowBinderNames_go(x_44, x_32, x_9); lean_dec(x_44); -x_47 = l_Lean_LocalDecl_userName(x_45); -lean_dec(x_45); -x_48 = l_Lean_Name_hasMacroScopes(x_47); -lean_dec(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; -x_49 = l_Lean_MessageData_ofExpr(x_2); -x_50 = l_Lean_Elab_Command_accLevelAtCtor___closed__8; -x_51 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_51, 0, x_50); -lean_ctor_set(x_51, 1, x_49); -x_52 = l_Lean_Elab_Command_accLevelAtCtor___closed__10; -x_53 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_53, 0, x_51); -lean_ctor_set(x_53, 1, x_52); -x_54 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_54, 0, x_43); -lean_ctor_set(x_54, 1, x_53); -x_55 = lean_box(0); -x_56 = l_Lean_Elab_Command_accLevelAtCtor___lambda__2(x_14, x_34, x_4, x_3, x_54, x_55, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_46); -return x_56; +lean_ctor_set(x_38, 0, x_45); +return x_38; } else { -lean_object* x_57; lean_object* x_58; -lean_dec(x_2); -x_57 = lean_box(0); -x_58 = l_Lean_Elab_Command_accLevelAtCtor___lambda__2(x_14, x_34, x_4, x_3, x_43, x_57, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_46); -return x_58; +lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_46 = lean_ctor_get(x_38, 0); +x_47 = lean_ctor_get(x_38, 1); +lean_inc(x_47); +lean_inc(x_46); +lean_dec(x_38); +x_48 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getArrowBinderNames(x_46); +x_49 = lean_array_get_size(x_25); +lean_dec(x_25); +x_50 = l_Array_toSubarray___rarg(x_48, x_9, x_49); +x_51 = l_Array_ofSubarray___rarg(x_50); +lean_dec(x_50); +x_52 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceArrowBinderNames_go(x_51, x_32, x_9); +lean_dec(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 { -uint8_t x_59; -lean_dec(x_43); -lean_dec(x_34); -lean_dec(x_14); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); +uint8_t x_54; +lean_dec(x_32); +lean_dec(x_25); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_59 = !lean_is_exclusive(x_44); -if (x_59 == 0) +x_54 = !lean_is_exclusive(x_35); +if (x_54 == 0) { -return x_44; +return x_35; } else { -lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_60 = lean_ctor_get(x_44, 0); -x_61 = lean_ctor_get(x_44, 1); -lean_inc(x_61); -lean_inc(x_60); -lean_dec(x_44); -x_62 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_62, 0, x_60); -lean_ctor_set(x_62, 1, x_61); -return x_62; +lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_55 = lean_ctor_get(x_35, 0); +x_56 = lean_ctor_get(x_35, 1); +lean_inc(x_56); +lean_inc(x_55); +lean_dec(x_35); +x_57 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_57, 0, x_55); +lean_ctor_set(x_57, 1, x_56); +return x_57; } } } else { -uint8_t x_63; -lean_free_object(x_27); -lean_free_object(x_23); -lean_free_object(x_19); -lean_dec(x_14); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); +uint8_t x_58; +lean_dec(x_25); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_63 = !lean_is_exclusive(x_33); -if (x_63 == 0) +x_58 = !lean_is_exclusive(x_31); +if (x_58 == 0) { -return x_33; +return x_31; } else { -lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_64 = lean_ctor_get(x_33, 0); -x_65 = lean_ctor_get(x_33, 1); -lean_inc(x_65); -lean_inc(x_64); -lean_dec(x_33); -x_66 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_66, 0, x_64); -lean_ctor_set(x_66, 1, x_65); -return x_66; +lean_object* x_59; lean_object* x_60; lean_object* x_61; +x_59 = lean_ctor_get(x_31, 0); +x_60 = lean_ctor_get(x_31, 1); +lean_inc(x_60); +lean_inc(x_59); +lean_dec(x_31); +x_61 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_61, 0, x_59); +lean_ctor_set(x_61, 1, x_60); +return x_61; } } } else { -uint8_t x_67; -lean_free_object(x_27); -lean_dec(x_29); -lean_free_object(x_23); -lean_free_object(x_19); -lean_dec(x_14); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); +lean_dec(x_25); +lean_dec(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); -lean_dec(x_1); -x_67 = !lean_is_exclusive(x_31); -if (x_67 == 0) -{ -lean_object* x_68; lean_object* x_69; -x_68 = lean_ctor_get(x_31, 0); -lean_dec(x_68); -x_69 = lean_box(0); -lean_ctor_set(x_31, 0, x_69); -return x_31; -} -else -{ -lean_object* x_70; lean_object* x_71; lean_object* x_72; -x_70 = lean_ctor_get(x_31, 1); -lean_inc(x_70); -lean_dec(x_31); -x_71 = lean_box(0); -x_72 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_72, 0, x_71); -lean_ctor_set(x_72, 1, x_70); -return x_72; -} +lean_ctor_set(x_20, 0, x_1); +return x_20; } } else { -lean_object* x_73; lean_object* x_74; lean_object* x_75; -x_73 = lean_ctor_get(x_27, 0); -x_74 = lean_ctor_get(x_27, 1); -lean_inc(x_74); +lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; uint8_t x_66; +x_62 = lean_ctor_get(x_20, 0); +x_63 = lean_ctor_get(x_20, 1); +lean_inc(x_63); +lean_inc(x_62); +lean_dec(x_20); +x_64 = lean_ctor_get(x_62, 0); +lean_inc(x_64); +x_65 = lean_ctor_get(x_62, 1); +lean_inc(x_65); +lean_dec(x_62); +x_66 = l_Array_isEmpty___rarg(x_65); +if (x_66 == 0) +{ +lean_object* x_67; uint8_t x_68; uint8_t x_69; uint8_t x_70; lean_object* x_71; +lean_dec(x_1); +lean_inc(x_65); +x_67 = l_Array_append___rarg(x_65, x_64); +lean_dec(x_64); +x_68 = 0; +x_69 = 1; +x_70 = 1; +lean_inc(x_3); +x_71 = l_Lean_Meta_mkForallFVars(x_67, x_3, x_68, x_69, x_70, x_4, x_5, x_6, x_7, x_63); +if (lean_obj_tag(x_71) == 0) +{ +lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; +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_27); -x_75 = lean_st_ref_set(x_5, x_74, x_26); -if (lean_obj_tag(x_73) == 0) +lean_dec(x_71); +x_74 = l_Lean_Expr_getAppFn(x_3); +lean_dec(x_3); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_75 = lean_infer_type(x_74, x_4, x_5, x_6, x_7, x_73); +if (lean_obj_tag(x_75) == 0) { -lean_object* x_76; lean_object* x_77; -x_76 = lean_ctor_get(x_75, 1); +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_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_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_14); -x_77 = lean_infer_type(x_14, x_8, x_9, x_10, x_11, x_76); -if (lean_obj_tag(x_77) == 0) -{ -lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; -x_78 = lean_ctor_get(x_77, 0); -lean_inc(x_78); -x_79 = lean_ctor_get(x_77, 1); +x_78 = l_Lean_instantiateMVars___at___private_Lean_Meta_Basic_0__Lean_Meta_isClassApp_x3f___spec__1(x_76, x_4, x_5, x_6, x_7, x_77); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_79 = lean_ctor_get(x_78, 0); lean_inc(x_79); -lean_dec(x_77); -x_80 = lean_ctor_get(x_1, 0); +x_80 = lean_ctor_get(x_78, 1); lean_inc(x_80); -x_81 = l_Lean_MessageData_ofName(x_80); -x_82 = l_Lean_Elab_Command_accLevelAtCtor___closed__2; -x_83 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_83, 0, x_82); -lean_ctor_set(x_83, 1, x_81); -x_84 = l_Lean_Elab_Command_accLevelAtCtor___closed__4; -lean_ctor_set_tag(x_23, 7); -lean_ctor_set(x_23, 1, x_84); -lean_ctor_set(x_23, 0, x_83); -x_85 = lean_ctor_get(x_1, 1); -lean_inc(x_85); -lean_dec(x_1); -x_86 = l_Lean_indentExpr(x_85); -lean_ctor_set_tag(x_19, 7); -lean_ctor_set(x_19, 1, x_86); -lean_ctor_set(x_19, 0, x_23); -x_87 = l_Lean_Elab_Command_accLevelAtCtor___closed__6; -x_88 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_88, 0, x_19); -lean_ctor_set(x_88, 1, x_87); -lean_inc(x_8); -x_89 = l_Lean_Meta_getFVarLocalDecl(x_2, x_8, x_9, x_10, x_11, x_79); -if (lean_obj_tag(x_89) == 0) -{ -lean_object* x_90; lean_object* x_91; lean_object* x_92; uint8_t x_93; -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_LocalDecl_userName(x_90); -lean_dec(x_90); -x_93 = l_Lean_Name_hasMacroScopes(x_92); -lean_dec(x_92); -if (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; -x_94 = l_Lean_MessageData_ofExpr(x_2); -x_95 = l_Lean_Elab_Command_accLevelAtCtor___closed__8; -x_96 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_96, 0, x_95); -lean_ctor_set(x_96, 1, x_94); -x_97 = l_Lean_Elab_Command_accLevelAtCtor___closed__10; -x_98 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_98, 0, x_96); -lean_ctor_set(x_98, 1, x_97); -x_99 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_99, 0, x_88); -lean_ctor_set(x_99, 1, x_98); -x_100 = lean_box(0); -x_101 = l_Lean_Elab_Command_accLevelAtCtor___lambda__2(x_14, x_78, x_4, x_3, x_99, x_100, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_91); -return x_101; +if (lean_is_exclusive(x_78)) { + lean_ctor_release(x_78, 0); + lean_ctor_release(x_78, 1); + x_81 = x_78; +} else { + lean_dec_ref(x_78); + x_81 = lean_box(0); } -else -{ -lean_object* x_102; lean_object* x_103; -lean_dec(x_2); -x_102 = lean_box(0); -x_103 = l_Lean_Elab_Command_accLevelAtCtor___lambda__2(x_14, x_78, x_4, x_3, x_88, x_102, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_91); -return x_103; +x_82 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getArrowBinderNames(x_79); +x_83 = lean_array_get_size(x_65); +lean_dec(x_65); +x_84 = l_Array_toSubarray___rarg(x_82, x_9, x_83); +x_85 = l_Array_ofSubarray___rarg(x_84); +lean_dec(x_84); +x_86 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceArrowBinderNames_go(x_85, x_72, x_9); +lean_dec(x_85); +if (lean_is_scalar(x_81)) { + x_87 = lean_alloc_ctor(0, 2, 0); +} else { + x_87 = x_81; } +lean_ctor_set(x_87, 0, x_86); +lean_ctor_set(x_87, 1, x_80); +return x_87; } else { -lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; -lean_dec(x_88); -lean_dec(x_78); -lean_dec(x_14); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); +lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; +lean_dec(x_72); +lean_dec(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_104 = lean_ctor_get(x_89, 0); -lean_inc(x_104); -x_105 = lean_ctor_get(x_89, 1); -lean_inc(x_105); -if (lean_is_exclusive(x_89)) { - lean_ctor_release(x_89, 0); - lean_ctor_release(x_89, 1); - x_106 = x_89; -} else { - lean_dec_ref(x_89); - x_106 = lean_box(0); +x_88 = lean_ctor_get(x_75, 0); +lean_inc(x_88); +x_89 = lean_ctor_get(x_75, 1); +lean_inc(x_89); +if (lean_is_exclusive(x_75)) { + lean_ctor_release(x_75, 0); + lean_ctor_release(x_75, 1); + x_90 = x_75; +} else { + lean_dec_ref(x_75); + x_90 = lean_box(0); } -if (lean_is_scalar(x_106)) { - x_107 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_90)) { + x_91 = lean_alloc_ctor(1, 2, 0); } else { - x_107 = x_106; + x_91 = x_90; } -lean_ctor_set(x_107, 0, x_104); -lean_ctor_set(x_107, 1, x_105); -return x_107; +lean_ctor_set(x_91, 0, x_88); +lean_ctor_set(x_91, 1, x_89); +return x_91; } } else { -lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; -lean_free_object(x_23); -lean_free_object(x_19); -lean_dec(x_14); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); +lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; +lean_dec(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); -lean_dec(x_1); -x_108 = lean_ctor_get(x_77, 0); -lean_inc(x_108); -x_109 = lean_ctor_get(x_77, 1); -lean_inc(x_109); -if (lean_is_exclusive(x_77)) { - lean_ctor_release(x_77, 0); - lean_ctor_release(x_77, 1); - x_110 = x_77; +x_92 = lean_ctor_get(x_71, 0); +lean_inc(x_92); +x_93 = lean_ctor_get(x_71, 1); +lean_inc(x_93); +if (lean_is_exclusive(x_71)) { + lean_ctor_release(x_71, 0); + lean_ctor_release(x_71, 1); + x_94 = x_71; } else { - lean_dec_ref(x_77); - x_110 = lean_box(0); + lean_dec_ref(x_71); + x_94 = lean_box(0); } -if (lean_is_scalar(x_110)) { - x_111 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_94)) { + x_95 = lean_alloc_ctor(1, 2, 0); } else { - x_111 = x_110; + x_95 = x_94; } -lean_ctor_set(x_111, 0, x_108); -lean_ctor_set(x_111, 1, x_109); -return x_111; +lean_ctor_set(x_95, 0, x_92); +lean_ctor_set(x_95, 1, x_93); +return x_95; } } else { -lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; -lean_dec(x_73); -lean_free_object(x_23); -lean_free_object(x_19); -lean_dec(x_14); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); +lean_object* x_96; +lean_dec(x_65); +lean_dec(x_64); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_112 = lean_ctor_get(x_75, 1); -lean_inc(x_112); -if (lean_is_exclusive(x_75)) { - lean_ctor_release(x_75, 0); - lean_ctor_release(x_75, 1); - x_113 = x_75; -} else { - lean_dec_ref(x_75); - x_113 = lean_box(0); -} -x_114 = lean_box(0); -if (lean_is_scalar(x_113)) { - x_115 = lean_alloc_ctor(0, 2, 0); -} else { - x_115 = x_113; -} -lean_ctor_set(x_115, 0, x_114); -lean_ctor_set(x_115, 1, x_112); -return x_115; +x_96 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_96, 0, x_1); +lean_ctor_set(x_96, 1, x_63); +return x_96; } } } else { -lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; -x_116 = lean_ctor_get(x_23, 0); -x_117 = lean_ctor_get(x_23, 1); -lean_inc(x_117); -lean_inc(x_116); -lean_dec(x_23); -lean_inc(x_4); -x_118 = l_Lean_Elab_Command_accLevel_go(x_3, x_21, x_4, x_116); -x_119 = lean_ctor_get(x_118, 0); -lean_inc(x_119); -x_120 = lean_ctor_get(x_118, 1); -lean_inc(x_120); -if (lean_is_exclusive(x_118)) { - lean_ctor_release(x_118, 0); - lean_ctor_release(x_118, 1); - x_121 = x_118; -} else { - lean_dec_ref(x_118); - x_121 = lean_box(0); -} -x_122 = lean_st_ref_set(x_5, x_120, x_117); -if (lean_obj_tag(x_119) == 0) -{ -lean_object* x_123; lean_object* x_124; -x_123 = lean_ctor_get(x_122, 1); -lean_inc(x_123); -lean_dec(x_122); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_14); -x_124 = lean_infer_type(x_14, x_8, x_9, x_10, x_11, x_123); -if (lean_obj_tag(x_124) == 0) +uint8_t x_97; +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_97 = !lean_is_exclusive(x_20); +if (x_97 == 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; lean_object* x_137; -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 = lean_ctor_get(x_1, 0); -lean_inc(x_127); -x_128 = l_Lean_MessageData_ofName(x_127); -x_129 = l_Lean_Elab_Command_accLevelAtCtor___closed__2; -if (lean_is_scalar(x_121)) { - x_130 = lean_alloc_ctor(7, 2, 0); -} else { - x_130 = x_121; - lean_ctor_set_tag(x_130, 7); +return x_20; } -lean_ctor_set(x_130, 0, x_129); -lean_ctor_set(x_130, 1, x_128); -x_131 = l_Lean_Elab_Command_accLevelAtCtor___closed__4; -x_132 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_132, 0, x_130); -lean_ctor_set(x_132, 1, x_131); -x_133 = lean_ctor_get(x_1, 1); -lean_inc(x_133); -lean_dec(x_1); -x_134 = l_Lean_indentExpr(x_133); -lean_ctor_set_tag(x_19, 7); -lean_ctor_set(x_19, 1, x_134); -lean_ctor_set(x_19, 0, x_132); -x_135 = l_Lean_Elab_Command_accLevelAtCtor___closed__6; -x_136 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_136, 0, x_19); -lean_ctor_set(x_136, 1, x_135); -lean_inc(x_8); -x_137 = l_Lean_Meta_getFVarLocalDecl(x_2, x_8, x_9, x_10, x_11, x_126); -if (lean_obj_tag(x_137) == 0) +else { -lean_object* x_138; lean_object* x_139; lean_object* x_140; uint8_t x_141; -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_LocalDecl_userName(x_138); -lean_dec(x_138); -x_141 = l_Lean_Name_hasMacroScopes(x_140); -lean_dec(x_140); -if (x_141 == 0) +lean_object* x_98; lean_object* x_99; lean_object* x_100; +x_98 = lean_ctor_get(x_20, 0); +x_99 = lean_ctor_get(x_20, 1); +lean_inc(x_99); +lean_inc(x_98); +lean_dec(x_20); +x_100 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_100, 0, x_98); +lean_ctor_set(x_100, 1, x_99); +return x_100; +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs(lean_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_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; -x_142 = l_Lean_MessageData_ofExpr(x_2); -x_143 = l_Lean_Elab_Command_accLevelAtCtor___closed__8; -x_144 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_144, 0, x_143); -lean_ctor_set(x_144, 1, x_142); -x_145 = l_Lean_Elab_Command_accLevelAtCtor___closed__10; -x_146 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_146, 0, x_144); -lean_ctor_set(x_146, 1, x_145); -x_147 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_147, 0, x_136); -lean_ctor_set(x_147, 1, x_146); -x_148 = lean_box(0); -x_149 = l_Lean_Elab_Command_accLevelAtCtor___lambda__2(x_14, x_125, x_4, x_3, x_147, x_148, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_139); -return x_149; +lean_object* x_7; uint8_t x_8; lean_object* x_9; +lean_inc(x_1); +x_7 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___lambda__1), 8, 1); +lean_closure_set(x_7, 0, x_1); +x_8 = 0; +x_9 = l_Lean_Meta_forallTelescopeReducing___at_Lean_Meta_getParamNames___spec__2___rarg(x_1, x_7, x_8, x_2, x_3, x_4, x_5, x_6); +return x_9; } -else +} +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: { -lean_object* x_150; lean_object* x_151; +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_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__1(x_1, x_2, x_5, x_6); lean_dec(x_2); -x_150 = lean_box(0); -x_151 = l_Lean_Elab_Command_accLevelAtCtor___lambda__2(x_14, x_125, x_4, x_3, x_136, x_150, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_139); -return x_151; +lean_dec(x_1); +x_8 = lean_box(x_7); +return x_8; } } -else +LEAN_EXPORT lean_object* l_Lean_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___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) { +_start: { -lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; -lean_dec(x_136); -lean_dec(x_125); -lean_dec(x_14); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); +lean_object* x_9; +x_9 = l_Lean_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_erase___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__3___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Array_erase___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__3(x_1, x_2); lean_dec(x_2); -x_152 = lean_ctor_get(x_137, 0); -lean_inc(x_152); -x_153 = lean_ctor_get(x_137, 1); -lean_inc(x_153); -if (lean_is_exclusive(x_137)) { - lean_ctor_release(x_137, 0); - lean_ctor_release(x_137, 1); - x_154 = x_137; -} else { - lean_dec_ref(x_137); - x_154 = lean_box(0); +return x_3; } -if (lean_is_scalar(x_154)) { - x_155 = lean_alloc_ctor(1, 2, 0); -} else { - x_155 = x_154; } -lean_ctor_set(x_155, 0, x_152); -lean_ctor_set(x_155, 1, x_153); -return x_155; +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* x_1, lean_object* x_2) { +_start: +{ +uint8_t x_3; lean_object* x_4; +x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__1(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +x_4 = lean_box(x_3); +return x_4; } } -else +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__2___boxed(lean_object* x_1) { +_start: { -lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; -lean_dec(x_121); -lean_free_object(x_19); -lean_dec(x_14); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); +uint8_t x_2; lean_object* x_3; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__2(x_1); +lean_dec(x_1); +x_3 = lean_box(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_156 = lean_ctor_get(x_124, 0); -lean_inc(x_156); -x_157 = lean_ctor_get(x_124, 1); -lean_inc(x_157); -if (lean_is_exclusive(x_124)) { - lean_ctor_release(x_124, 0); - lean_ctor_release(x_124, 1); - x_158 = x_124; -} else { - lean_dec_ref(x_124); - x_158 = lean_box(0); +return x_10; } -if (lean_is_scalar(x_158)) { - x_159 = lean_alloc_ctor(1, 2, 0); -} else { - x_159 = x_158; } -lean_ctor_set(x_159, 0, x_156); -lean_ctor_set(x_159, 1, x_157); -return x_159; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__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); +lean_dec(x_6); +lean_dec(x_5); +return x_11; } } -else +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: { -lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; -lean_dec(x_121); -lean_dec(x_119); -lean_free_object(x_19); -lean_dec(x_14); -lean_dec(x_11); -lean_dec(x_10); +lean_object* x_11; +x_11 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__5(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_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__6(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_4); -lean_dec(x_3); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___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) { +_start: +{ +size_t x_10; size_t x_11; lean_object* x_12; +x_10 = lean_unbox_usize(x_2); lean_dec(x_2); +x_11 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_12 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4(x_1, x_10, x_11, 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_1); -x_160 = lean_ctor_get(x_122, 1); -lean_inc(x_160); -if (lean_is_exclusive(x_122)) { - lean_ctor_release(x_122, 0); - lean_ctor_release(x_122, 1); - x_161 = x_122; -} else { - lean_dec_ref(x_122); - x_161 = lean_box(0); -} -x_162 = lean_box(0); -if (lean_is_scalar(x_161)) { - x_163 = lean_alloc_ctor(0, 2, 0); -} else { - x_163 = x_161; +return x_12; } -lean_ctor_set(x_163, 0, x_162); -lean_ctor_set(x_163, 1, x_160); -return x_163; } +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___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_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; +x_14 = lean_array_uget(x_1, x_3); +lean_inc(x_7); +x_15 = l_Lean_Meta_getFVarLocalDecl(x_14, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_15) == 0) +{ +lean_object* x_16; lean_object* x_17; uint8_t x_18; uint8_t 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 = l_Lean_LocalDecl_binderInfo(x_16); +lean_dec(x_16); +x_19 = l_Lean_BinderInfo_isExplicit(x_18); +if (x_19 == 0) +{ +size_t x_20; size_t x_21; +lean_dec(x_14); +x_20 = 1; +x_21 = lean_usize_add(x_3, x_20); +x_3 = x_21; +x_11 = x_17; +goto _start; } else { -lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; -x_164 = lean_ctor_get(x_19, 0); -x_165 = lean_ctor_get(x_19, 1); -lean_inc(x_165); -lean_inc(x_164); -lean_dec(x_19); -x_166 = lean_st_ref_take(x_5, x_165); -x_167 = lean_ctor_get(x_166, 0); -lean_inc(x_167); -x_168 = lean_ctor_get(x_166, 1); -lean_inc(x_168); -if (lean_is_exclusive(x_166)) { - lean_ctor_release(x_166, 0); - lean_ctor_release(x_166, 1); - x_169 = x_166; -} else { - lean_dec_ref(x_166); - x_169 = lean_box(0); +lean_object* x_23; uint8_t x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; size_t x_28; size_t x_29; +x_23 = l_Lean_Expr_fvarId_x21(x_14); +lean_dec(x_14); +x_24 = 1; +x_25 = lean_box(x_24); +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_27 = lean_array_push(x_4, x_26); +x_28 = 1; +x_29 = lean_usize_add(x_3, x_28); +x_3 = x_29; +x_4 = x_27; +x_11 = x_17; +goto _start; } -lean_inc(x_4); -x_170 = l_Lean_Elab_Command_accLevel_go(x_3, x_164, x_4, x_167); -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; -} else { - lean_dec_ref(x_170); - x_173 = lean_box(0); } -x_174 = lean_st_ref_set(x_5, x_172, x_168); -if (lean_obj_tag(x_171) == 0) +else { -lean_object* x_175; lean_object* x_176; -x_175 = lean_ctor_get(x_174, 1); -lean_inc(x_175); -lean_dec(x_174); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_14); -x_176 = lean_infer_type(x_14, x_8, x_9, x_10, x_11, x_175); -if (lean_obj_tag(x_176) == 0) -{ -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; -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_ctor_get(x_1, 0); -lean_inc(x_179); -x_180 = l_Lean_MessageData_ofName(x_179); -x_181 = l_Lean_Elab_Command_accLevelAtCtor___closed__2; -if (lean_is_scalar(x_173)) { - x_182 = lean_alloc_ctor(7, 2, 0); -} else { - x_182 = x_173; - lean_ctor_set_tag(x_182, 7); -} -lean_ctor_set(x_182, 0, x_181); -lean_ctor_set(x_182, 1, x_180); -x_183 = l_Lean_Elab_Command_accLevelAtCtor___closed__4; -if (lean_is_scalar(x_169)) { - x_184 = lean_alloc_ctor(7, 2, 0); -} else { - x_184 = x_169; - lean_ctor_set_tag(x_184, 7); -} -lean_ctor_set(x_184, 0, x_182); -lean_ctor_set(x_184, 1, x_183); -x_185 = lean_ctor_get(x_1, 1); -lean_inc(x_185); -lean_dec(x_1); -x_186 = l_Lean_indentExpr(x_185); -x_187 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_187, 0, x_184); -lean_ctor_set(x_187, 1, x_186); -x_188 = l_Lean_Elab_Command_accLevelAtCtor___closed__6; -x_189 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_189, 0, x_187); -lean_ctor_set(x_189, 1, x_188); -lean_inc(x_8); -x_190 = l_Lean_Meta_getFVarLocalDecl(x_2, x_8, x_9, x_10, x_11, x_178); -if (lean_obj_tag(x_190) == 0) -{ -lean_object* x_191; lean_object* x_192; lean_object* x_193; uint8_t x_194; -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_LocalDecl_userName(x_191); -lean_dec(x_191); -x_194 = l_Lean_Name_hasMacroScopes(x_193); -lean_dec(x_193); -if (x_194 == 0) +uint8_t x_31; +lean_dec(x_14); +lean_dec(x_7); +lean_dec(x_4); +x_31 = !lean_is_exclusive(x_15); +if (x_31 == 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; -x_195 = l_Lean_MessageData_ofExpr(x_2); -x_196 = l_Lean_Elab_Command_accLevelAtCtor___closed__8; -x_197 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_197, 0, x_196); -lean_ctor_set(x_197, 1, x_195); -x_198 = l_Lean_Elab_Command_accLevelAtCtor___closed__10; -x_199 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_199, 0, x_197); -lean_ctor_set(x_199, 1, x_198); -x_200 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_200, 0, x_189); -lean_ctor_set(x_200, 1, x_199); -x_201 = lean_box(0); -x_202 = l_Lean_Elab_Command_accLevelAtCtor___lambda__2(x_14, x_177, x_4, x_3, x_200, x_201, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_192); -return x_202; +return x_15; } else { -lean_object* x_203; lean_object* x_204; -lean_dec(x_2); -x_203 = lean_box(0); -x_204 = l_Lean_Elab_Command_accLevelAtCtor___lambda__2(x_14, x_177, x_4, x_3, x_189, x_203, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_192); -return x_204; +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_15, 0); +x_33 = lean_ctor_get(x_15, 1); +lean_inc(x_33); +lean_inc(x_32); +lean_dec(x_15); +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_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; -lean_dec(x_189); -lean_dec(x_177); -lean_dec(x_14); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_205 = lean_ctor_get(x_190, 0); -lean_inc(x_205); -x_206 = lean_ctor_get(x_190, 1); -lean_inc(x_206); -if (lean_is_exclusive(x_190)) { - lean_ctor_release(x_190, 0); - lean_ctor_release(x_190, 1); - x_207 = x_190; -} else { - lean_dec_ref(x_190); - x_207 = lean_box(0); } -if (lean_is_scalar(x_207)) { - x_208 = lean_alloc_ctor(1, 2, 0); -} else { - x_208 = x_207; } -lean_ctor_set(x_208, 0, x_205); -lean_ctor_set(x_208, 1, x_206); -return x_208; } +LEAN_EXPORT lean_object* l_Lean_Meta_withNewBinderInfos___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; +x_10 = lean_apply_2(x_2, x_3, x_4); +x_11 = l___private_Lean_Meta_Basic_0__Lean_Meta_withNewBinderInfosImp___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_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; -lean_dec(x_173); -lean_dec(x_169); -lean_dec(x_14); +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); -lean_dec(x_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_209 = lean_ctor_get(x_176, 0); -lean_inc(x_209); -x_210 = lean_ctor_get(x_176, 1); -lean_inc(x_210); -if (lean_is_exclusive(x_176)) { - lean_ctor_release(x_176, 0); - lean_ctor_release(x_176, 1); - x_211 = x_176; -} else { - lean_dec_ref(x_176); - x_211 = lean_box(0); -} -if (lean_is_scalar(x_211)) { - x_212 = lean_alloc_ctor(1, 2, 0); -} else { - x_212 = x_211; +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_ctor_set(x_212, 0, x_209); -lean_ctor_set(x_212, 1, x_210); -return x_212; } +else +{ +uint8_t x_16; +x_16 = !lean_is_exclusive(x_11); +if (x_16 == 0) +{ +return x_11; } else { -lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; -lean_dec(x_173); -lean_dec(x_171); -lean_dec(x_169); -lean_dec(x_14); +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); -lean_dec(x_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_213 = lean_ctor_get(x_174, 1); -lean_inc(x_213); -if (lean_is_exclusive(x_174)) { - lean_ctor_release(x_174, 0); - lean_ctor_release(x_174, 1); - x_214 = x_174; -} else { - lean_dec_ref(x_174); - x_214 = 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); +return x_19; +} } -x_215 = lean_box(0); -if (lean_is_scalar(x_214)) { - x_216 = lean_alloc_ctor(0, 2, 0); -} else { - x_216 = x_214; } -lean_ctor_set(x_216, 0, x_215); -lean_ctor_set(x_216, 1, x_213); -return x_216; } +LEAN_EXPORT lean_object* l_Lean_Meta_withNewBinderInfos___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___spec__2(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withNewBinderInfos___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___spec__2___rarg___boxed), 9, 0); +return x_2; } } -else +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___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_217; -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_217 = !lean_is_exclusive(x_16); -if (x_217 == 0) +size_t x_10; size_t x_11; lean_object* x_12; lean_object* x_13; +x_10 = lean_array_size(x_1); +x_11 = 0; +x_12 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__8___closed__1; +lean_inc(x_5); +x_13 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___spec__1(x_1, x_10, x_11, x_12, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_13) == 0) { +lean_object* x_14; lean_object* x_15; 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_Lean_Meta_withNewBinderInfos___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___spec__2___rarg(x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_15); +lean_dec(x_14); return x_16; } else { -lean_object* x_218; lean_object* x_219; lean_object* x_220; -x_218 = lean_ctor_get(x_16, 0); -x_219 = lean_ctor_get(x_16, 1); -lean_inc(x_219); -lean_inc(x_218); -lean_dec(x_16); -x_220 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_220, 0, x_218); -lean_ctor_set(x_220, 1, x_219); -return x_220; -} -} -} -else -{ -uint8_t x_221; -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); +uint8_t x_17; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -13170,705 +13851,723 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_221 = !lean_is_exclusive(x_13); -if (x_221 == 0) +x_17 = !lean_is_exclusive(x_13); +if (x_17 == 0) { return x_13; } else { -lean_object* x_222; lean_object* x_223; lean_object* x_224; -x_222 = lean_ctor_get(x_13, 0); -x_223 = lean_ctor_get(x_13, 1); -lean_inc(x_223); -lean_inc(x_222); +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_13, 0); +x_19 = lean_ctor_get(x_13, 1); +lean_inc(x_19); +lean_inc(x_18); lean_dec(x_13); -x_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_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_instantiateLevelMVars___at_Lean_Elab_Command_accLevelAtCtor___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_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit(lean_object* x_1) { _start: { -lean_object* x_10; -x_10 = l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_accLevelAtCtor___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_10; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___rarg___boxed), 9, 0); +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_accLevelAtCtor___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___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_10; -x_10 = l_Lean_throwError___at_Lean_Elab_Command_accLevelAtCtor___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); +size_t x_12; size_t x_13; lean_object* x_14; +x_12 = lean_unbox_usize(x_2); lean_dec(x_2); -return x_10; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Command_accLevelAtCtor___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, 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_Command_accLevelAtCtor___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_13 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_14 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___spec__1(x_1, x_12, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_11; +lean_dec(x_1); +return x_14; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_accLevelAtCtor___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_Meta_withNewBinderInfos___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___spec__2___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_15; -x_15 = l_Lean_Elab_Command_accLevelAtCtor___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; +lean_object* x_10; +x_10 = l_Lean_Meta_withNewBinderInfos___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___spec__2___rarg(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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___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, lean_object* x_7, lean_object* x_8, size_t x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___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) { _start: { -if (lean_obj_tag(x_10) == 0) -{ -lean_object* x_11; lean_object* 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); -lean_dec(x_3); -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -lean_dec(x_10); -x_12 = lean_ctor_get(x_1, 0); -lean_inc(x_12); +lean_object* x_10; +x_10 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_1); -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_11); -return x_14; +return x_10; } -else +} +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___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_15; size_t x_16; size_t x_17; lean_object* x_18; -x_15 = lean_ctor_get(x_10, 0); -lean_inc(x_15); -lean_dec(x_10); -x_16 = 1; -x_17 = lean_usize_add(x_2, x_16); -x_18 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_17, x_15); -return x_18; +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_array_set(x_3, x_1, x_2); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_11); +lean_ctor_set(x_12, 1, x_9); +return x_12; +} } +static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___spec__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("inductive datatype parameter mismatch", 37, 37); +return x_1; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___spec__1___closed__2() { _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; lean_object* x_2; +x_1 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___spec__1___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___spec__1___closed__3() { _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_object* x_1; +x_1 = lean_mk_string_unchecked("\nexpected", 9, 9); +return x_1; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg___lambda__4(lean_object* x_1, lean_object* x_2) { +static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___spec__1___closed__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; -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_box(0); -x_7 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_7, 0, x_5); -lean_ctor_set(x_7, 1, x_6); -x_8 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_8, 0, x_7); -x_9 = lean_apply_2(x_4, lean_box(0), x_8); -return x_9; +lean_object* x_1; lean_object* x_2; +x_1 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___spec__1___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, size_t x_8, size_t x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___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: { -uint8_t x_11; -x_11 = lean_usize_dec_lt(x_9, x_8); -if (x_11 == 0) +uint8_t x_13; +x_13 = lean_nat_dec_le(x_5, x_4); +if (x_13 == 0) { -lean_object* 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); +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_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; uint8_t x_20; lean_object* x_21; +x_16 = lean_unsigned_to_nat(1u); +x_17 = lean_nat_sub(x_3, x_16); lean_dec(x_3); -lean_dec(x_2); -x_12 = lean_ctor_get(x_1, 0); -lean_inc(x_12); -lean_dec(x_1); -x_13 = lean_ctor_get(x_12, 1); -lean_inc(x_13); -lean_dec(x_12); -x_14 = lean_apply_2(x_13, lean_box(0), x_10); -return x_14; +x_18 = lean_nat_dec_lt(x_4, x_2); +x_19 = lean_array_get_size(x_7); +x_20 = lean_nat_dec_lt(x_4, x_19); +lean_dec(x_19); +if (x_18 == 0) +{ +lean_object* x_58; lean_object* x_59; +x_58 = l_Lean_instInhabitedExpr; +x_59 = l_outOfBounds___rarg(x_58); +x_21 = x_59; +goto block_57; } else { -lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -lean_dec(x_10); -x_15 = lean_array_uget(x_7, x_9); -x_16 = lean_ctor_get(x_1, 1); -lean_inc(x_16); -x_17 = lean_ctor_get(x_15, 2); -lean_inc(x_17); -x_18 = lean_name_eq(x_17, x_3); -lean_dec(x_17); -x_19 = lean_box_usize(x_9); -x_20 = lean_box_usize(x_8); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_2); -lean_inc(x_1); -x_21 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg___lambda__1___boxed), 10, 9); -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_6); -lean_closure_set(x_21, 7, x_7); -lean_closure_set(x_21, 8, x_20); -if (x_18 == 0) +lean_object* x_60; +x_60 = lean_array_fget(x_1, x_4); +x_21 = x_60; +goto block_57; +} +block_57: { -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_15); -lean_dec(x_4); -lean_dec(x_2); -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 = lean_box(0); -lean_inc(x_23); -x_25 = lean_apply_2(x_23, lean_box(0), x_24); -x_26 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg___lambda__2___boxed), 3, 2); -lean_closure_set(x_26, 0, x_6); -lean_closure_set(x_26, 1, x_23); -x_27 = lean_apply_4(x_5, lean_box(0), lean_box(0), x_25, x_26); -x_28 = lean_apply_4(x_16, lean_box(0), lean_box(0), x_27, x_21); -return x_28; +lean_object* x_22; +if (x_20 == 0) +{ +lean_object* x_54; lean_object* x_55; +x_54 = l_Lean_instInhabitedExpr; +x_55 = l_outOfBounds___rarg(x_54); +x_22 = x_55; +goto block_53; } 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_dec(x_6); -x_29 = lean_ctor_get(x_15, 0); -lean_inc(x_29); -lean_dec(x_15); -x_30 = lean_ctor_get(x_2, 0); -lean_inc(x_30); -x_31 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg___lambda__3___boxed), 4, 3); -lean_closure_set(x_31, 0, x_29); -lean_closure_set(x_31, 1, x_2); -lean_closure_set(x_31, 2, x_4); -lean_inc(x_5); -x_32 = lean_apply_4(x_5, lean_box(0), lean_box(0), x_30, x_31); -x_33 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg___lambda__4), 2, 1); -lean_closure_set(x_33, 0, x_1); -x_34 = lean_apply_4(x_5, lean_box(0), lean_box(0), x_32, x_33); -x_35 = lean_apply_4(x_16, lean_box(0), lean_box(0), x_34, x_21); -return x_35; -} -} -} +lean_object* x_56; +x_56 = lean_array_fget(x_7, x_4); +x_22 = x_56; +goto block_53; } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1(lean_object* x_1, lean_object* x_2) { -_start: +block_53: { -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg___boxed), 10, 0); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__2___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: +lean_object* x_23; +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_22); +lean_inc(x_21); +x_23 = l_Lean_Meta_isExprDefEq(x_21, x_22, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_23) == 0) { -lean_object* x_5; -x_5 = lean_ctor_get(x_4, 0); -lean_inc(x_5); +lean_object* x_24; uint8_t x_25; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_unbox(x_24); +lean_dec(x_24); +if (x_25 == 0) +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; +lean_dec(x_17); +lean_dec(x_7); lean_dec(x_4); -if (lean_obj_tag(x_5) == 0) +x_26 = lean_ctor_get(x_23, 1); +lean_inc(x_26); +lean_dec(x_23); +x_27 = l_Lean_indentExpr(x_22); +x_28 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___spec__1___closed__2; +x_29 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_27); +x_30 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___spec__1___closed__4; +x_31 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_31, 0, x_29); +lean_ctor_set(x_31, 1, x_30); +x_32 = l_Lean_indentExpr(x_21); +x_33 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_33, 0, x_31); +lean_ctor_set(x_33, 1, x_32); +x_34 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +x_35 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +x_36 = l_Lean_throwError___at_Lean_Meta_mkSimpCongrTheorem___spec__4(x_35, x_8, x_9, x_10, x_11, x_26); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +x_37 = !lean_is_exclusive(x_36); +if (x_37 == 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; -x_6 = lean_ctor_get(x_1, 0); -lean_inc(x_6); -lean_dec(x_1); -x_7 = lean_ctor_get(x_6, 1); -lean_inc(x_7); -lean_dec(x_6); -x_8 = lean_box(0); -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_Command_withCtorRef___spec__1___rarg___lambda__2___boxed), 3, 2); -lean_closure_set(x_10, 0, x_2); -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; +return x_36; } else { -uint8_t x_12; -lean_dec(x_3); -lean_dec(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; lean_object* x_18; -x_13 = lean_ctor_get(x_1, 0); -lean_inc(x_13); -lean_dec(x_1); -x_14 = lean_ctor_get(x_13, 1); -lean_inc(x_14); -lean_dec(x_13); -x_15 = lean_box(0); -x_16 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_16, 0, x_5); -lean_ctor_set(x_16, 1, x_15); -x_17 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_17, 0, x_16); -x_18 = lean_apply_2(x_14, lean_box(0), x_17); -return x_18; +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; +} } else { -lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_19 = lean_ctor_get(x_5, 0); -lean_inc(x_19); -lean_dec(x_5); -x_20 = lean_ctor_get(x_1, 0); -lean_inc(x_20); -lean_dec(x_1); -x_21 = lean_ctor_get(x_20, 1); -lean_inc(x_21); -lean_dec(x_20); -x_22 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_22, 0, x_19); -x_23 = lean_box(0); -x_24 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_24, 0, x_22); -lean_ctor_set(x_24, 1, x_23); -x_25 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_25, 0, x_24); -x_26 = lean_apply_2(x_21, lean_box(0), x_25); -return x_26; -} -} +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_22); +x_41 = lean_ctor_get(x_23, 1); +lean_inc(x_41); +lean_dec(x_23); +x_42 = lean_box(0); +x_43 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___spec__1___lambda__1(x_4, x_21, x_7, x_42, x_8, x_9, x_10, x_11, x_41); +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_ctor_get(x_44, 0); +lean_inc(x_46); +lean_dec(x_44); +x_47 = lean_nat_add(x_4, x_6); +lean_dec(x_4); +x_3 = x_17; +x_4 = x_47; +x_7 = x_46; +x_12 = x_45; +goto _start; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__2___rarg___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, size_t x_9, lean_object* x_10) { -_start: -{ -if (lean_obj_tag(x_10) == 0) +else { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +uint8_t x_49; +lean_dec(x_22); +lean_dec(x_21); +lean_dec(x_17); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -lean_dec(x_10); -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_apply_2(x_13, lean_box(0), x_11); -return x_14; +x_49 = !lean_is_exclusive(x_23); +if (x_49 == 0) +{ +return x_23; } else { -lean_object* x_15; size_t x_16; size_t x_17; lean_object* x_18; -x_15 = lean_ctor_get(x_10, 0); -lean_inc(x_15); -lean_dec(x_10); -x_16 = 1; -x_17 = lean_usize_add(x_2, x_16); -x_18 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__2___rarg(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_17, x_15); -return x_18; +lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_50 = lean_ctor_get(x_23, 0); +x_51 = lean_ctor_get(x_23, 1); +lean_inc(x_51); +lean_inc(x_50); +lean_dec(x_23); +x_52 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_52, 0, x_50); +lean_ctor_set(x_52, 1, x_51); +return x_52; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, size_t x_8, size_t x_9, lean_object* x_10) { -_start: -{ -uint8_t x_11; -x_11 = lean_usize_dec_lt(x_9, x_8); -if (x_11 == 0) +} +} +else { -lean_object* x_12; lean_object* x_13; lean_object* x_14; -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); +lean_object* x_61; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); -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_apply_2(x_13, lean_box(0), x_10); -return x_14; +x_61 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_61, 0, x_7); +lean_ctor_set(x_61, 1, x_12); +return x_61; +} } else { -lean_object* x_15; lean_object* x_16; lean_object* x_17; size_t x_18; size_t x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +lean_object* x_62; +lean_dec(x_11); lean_dec(x_10); -x_15 = lean_array_uget(x_7, x_9); -x_16 = lean_ctor_get(x_1, 1); -lean_inc(x_16); -x_17 = lean_ctor_get(x_15, 8); -lean_inc(x_17); -lean_dec(x_15); -x_18 = lean_array_size(x_17); -x_19 = 0; -lean_inc_n(x_6, 2); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_2); -lean_inc(x_1); -x_20 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_17, x_18, x_19, x_6); -lean_inc(x_5); -lean_inc(x_6); -lean_inc(x_1); -x_21 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__2___rarg___lambda__1), 4, 3); -lean_closure_set(x_21, 0, x_1); -lean_closure_set(x_21, 1, x_6); -lean_closure_set(x_21, 2, x_5); -lean_inc(x_5); -x_22 = lean_apply_4(x_5, lean_box(0), lean_box(0), x_20, x_21); -x_23 = lean_box_usize(x_9); -x_24 = lean_box_usize(x_8); -x_25 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__2___rarg___lambda__2___boxed), 10, 9); -lean_closure_set(x_25, 0, x_1); -lean_closure_set(x_25, 1, x_23); -lean_closure_set(x_25, 2, x_2); -lean_closure_set(x_25, 3, x_3); -lean_closure_set(x_25, 4, x_4); -lean_closure_set(x_25, 5, x_5); -lean_closure_set(x_25, 6, x_6); -lean_closure_set(x_25, 7, x_7); -lean_closure_set(x_25, 8, x_24); -x_26 = lean_apply_4(x_16, lean_box(0), lean_box(0), x_22, x_25); -return x_26; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_4); +lean_dec(x_3); +x_62 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_62, 0, x_7); +lean_ctor_set(x_62, 1, x_12); +return x_62; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__2(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___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_3; -x_3 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__2___rarg___boxed), 10, 0); -return x_3; -} +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_10 = lean_array_get_size(x_1); +x_11 = lean_unsigned_to_nat(0u); +x_12 = lean_unsigned_to_nat(1u); +lean_inc(x_10); +x_13 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___spec__1(x_1, x_10, x_10, x_11, x_10, x_12, x_3, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_10); +if (lean_obj_tag(x_13) == 0) +{ +uint8_t x_14; +x_14 = !lean_is_exclusive(x_13); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_15 = lean_ctor_get(x_13, 0); +x_16 = l_Lean_mkAppN(x_2, x_15); +lean_dec(x_15); +x_17 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_17, 0, x_16); +lean_ctor_set(x_13, 0, x_17); +return x_13; } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_withCtorRef___rarg___lambda__1(lean_object* x_1, lean_object* x_2) { -_start: +else { -lean_inc(x_1); -return x_1; +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_13, 0); +x_19 = lean_ctor_get(x_13, 1); +lean_inc(x_19); +lean_inc(x_18); +lean_dec(x_13); +x_20 = l_Lean_mkAppN(x_2, x_18); +lean_dec(x_18); +x_21 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_21, 0, x_20); +x_22 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_22, 0, x_21); +lean_ctor_set(x_22, 1, x_19); +return x_22; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_withCtorRef___rarg___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 = lean_ctor_get(x_4, 0); -lean_inc(x_5); -lean_dec(x_4); -if (lean_obj_tag(x_5) == 0) +else { -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_6 = lean_alloc_closure((void*)(l_Lean_Elab_Command_withCtorRef___rarg___lambda__1___boxed), 2, 1); -lean_closure_set(x_6, 0, x_1); -x_7 = lean_ctor_get(x_2, 0); -lean_inc(x_7); +uint8_t x_23; lean_dec(x_2); -x_8 = lean_ctor_get(x_7, 1); -lean_inc(x_8); -lean_dec(x_7); -x_9 = lean_box(0); -x_10 = lean_apply_2(x_8, lean_box(0), x_9); -x_11 = lean_apply_4(x_3, lean_box(0), lean_box(0), x_10, x_6); -return x_11; +x_23 = !lean_is_exclusive(x_13); +if (x_23 == 0) +{ +return x_13; } else { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -lean_dec(x_3); -lean_dec(x_1); -x_12 = lean_ctor_get(x_5, 0); -lean_inc(x_12); -lean_dec(x_5); -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_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_13, 0); +x_25 = lean_ctor_get(x_13, 1); +lean_inc(x_25); +lean_inc(x_24); lean_dec(x_13); -x_15 = lean_apply_2(x_14, lean_box(0), x_12); -return x_15; +x_26 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_26, 0, x_24); +lean_ctor_set(x_26, 1, x_25); +return x_26; } } } -static lean_object* _init_l_Lean_Elab_Command_withCtorRef___rarg___closed__1() { +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___lambda__2___closed__1() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; +lean_object* x_1; lean_object* x_2; 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; +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_Elab_Command_withCtorRef___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_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___lambda__2___closed__2() { _start: { -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; -x_6 = lean_ctor_get(x_1, 1); -lean_inc(x_6); -x_7 = lean_array_size(x_3); -x_8 = 0; -x_9 = l_Lean_Elab_Command_withCtorRef___rarg___closed__1; -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_1); -x_10 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__2___rarg(x_1, x_2, x_4, x_5, x_6, x_9, x_3, x_7, x_8, x_9); -lean_inc(x_6); -x_11 = lean_alloc_closure((void*)(l_Lean_Elab_Command_withCtorRef___rarg___lambda__2), 4, 3); -lean_closure_set(x_11, 0, x_5); -lean_closure_set(x_11, 1, x_1); -lean_closure_set(x_11, 2, 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 = lean_mk_string_unchecked("unexpected inductive type occurrence", 36, 36); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_withCtorRef(lean_object* x_1, lean_object* x_2) { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___lambda__2___closed__3() { _start: { -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Lean_Elab_Command_withCtorRef___rarg), 5, 0); -return x_3; +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___lambda__2___closed__2; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -size_t x_11; size_t x_12; lean_object* x_13; -x_11 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_12 = lean_unbox_usize(x_9); +lean_object* x_9; uint8_t x_10; +x_9 = l_Lean_Expr_getAppFn(x_3); +x_10 = l_Array_contains___at_Lean_Meta_setMVarUserNamesAt___spec__1(x_1, x_9); +if (x_10 == 0) +{ +lean_object* x_11; lean_object* x_12; lean_dec(x_9); -x_13 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg___lambda__1(x_1, x_11, x_3, x_4, x_5, x_6, x_7, x_8, x_12, x_10); -return x_13; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___lambda__2___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_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; uint8_t x_22; +x_13 = lean_unsigned_to_nat(0u); +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); +x_17 = lean_unsigned_to_nat(1u); +x_18 = lean_nat_sub(x_14, x_17); +lean_dec(x_14); +lean_inc(x_3); +x_19 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_3, x_16, x_18); +x_20 = lean_array_get_size(x_2); +x_21 = lean_array_get_size(x_19); +x_22 = lean_nat_dec_le(x_20, x_21); +lean_dec(x_21); +lean_dec(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; uint8_t x_29; +lean_dec(x_19); +lean_dec(x_9); +x_23 = l_Lean_indentExpr(x_3); +x_24 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___lambda__2___closed__3; +x_25 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_25, 0, x_24); +lean_ctor_set(x_25, 1, x_23); +x_26 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +x_27 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +x_28 = l_Lean_throwError___at_Lean_Meta_mkSimpCongrTheorem___spec__4(x_27, 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_29 = !lean_is_exclusive(x_28); +if (x_29 == 0) +{ +return x_28; } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: +else { -lean_object* x_4; -x_4 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg___lambda__2(x_1, x_2, x_3); +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_28, 0); +x_31 = lean_ctor_get(x_28, 1); +lean_inc(x_31); +lean_inc(x_30); +lean_dec(x_28); +x_32 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_31); +return x_32; +} +} +else +{ +lean_object* x_33; lean_object* x_34; lean_dec(x_3); -return x_4; +x_33 = lean_box(0); +x_34 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___lambda__1(x_2, x_9, x_19, x_33, x_4, x_5, x_6, x_7, x_8); +return x_34; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___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_5; -x_5 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg___lambda__3(x_1, x_2, x_3, x_4); -lean_dec(x_4); -lean_dec(x_1); -return x_5; +lean_object* x_7; lean_object* x_8; +x_7 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_7, 0, x_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); +return x_8; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___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) { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___closed__1() { _start: { -size_t x_11; size_t x_12; lean_object* x_13; -x_11 = lean_unbox_usize(x_8); +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___lambda__3___boxed), 6, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; lean_object* x_10; uint8_t x_11; lean_object* x_12; +x_9 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___lambda__2___boxed), 8, 2); +lean_closure_set(x_9, 0, x_1); +lean_closure_set(x_9, 1, x_2); +x_10 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___closed__1; +x_11 = 0; +x_12 = l_Lean_Meta_transform___at_Lean_Meta_zetaReduce___spec__1(x_3, x_9, x_10, x_11, x_11, x_4, x_5, x_6, x_7, x_8); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_8); -x_12 = lean_unbox_usize(x_9); -lean_dec(x_9); -x_13 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_11, x_12, x_10); -return x_13; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_1); +return x_10; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___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) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___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_11; size_t x_12; lean_object* x_13; -x_11 = lean_unbox_usize(x_2); +lean_object* x_13; +x_13 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_6); +lean_dec(x_5); lean_dec(x_2); -x_12 = lean_unbox_usize(x_9); -lean_dec(x_9); -x_13 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__2___rarg___lambda__2(x_1, x_11, x_3, x_4, x_5, x_6, x_7, x_8, x_12, x_10); +lean_dec(x_1); return x_13; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__2___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, 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_11; size_t x_12; lean_object* x_13; -x_11 = lean_unbox_usize(x_8); -lean_dec(x_8); -x_12 = lean_unbox_usize(x_9); -lean_dec(x_9); -x_13 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__2___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_11, x_12, x_10); -return x_13; +lean_object* x_10; +x_10 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___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_1); +return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_withCtorRef___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_3; -x_3 = l_Lean_Elab_Command_withCtorRef___rarg___lambda__1(x_1, x_2); +lean_object* x_9; +x_9 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_2); lean_dec(x_1); -return x_3; +return x_9; } } -LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___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: { -uint8_t x_16; -x_16 = lean_usize_dec_lt(x_6, x_5); -if (x_16 == 0) +lean_object* x_7; +x_7 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___lambda__3(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_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___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_17; -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); +lean_object* x_12; lean_object* x_13; +x_12 = l_Lean_mkAppN(x_1, x_2); +x_13 = lean_apply_8(x_3, x_12, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_13; +} +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__2___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("unexpected constructor resulting type, type expected", 52, 52); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__2___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__2___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___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_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_1); +x_10 = l_Lean_Meta_isType(x_1, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_10) == 0) +{ +lean_object* x_11; uint8_t x_12; +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +x_12 = lean_unbox(x_11); lean_dec(x_11); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_13 = lean_ctor_get(x_10, 1); +lean_inc(x_13); lean_dec(x_10); -lean_dec(x_9); +x_14 = l_Lean_indentExpr(x_1); +x_15 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__2___closed__2; +x_16 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_16, 1, x_14); +x_17 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +x_18 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_18, 0, x_16); +lean_ctor_set(x_18, 1, x_17); +x_19 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_18, x_3, x_4, x_5, x_6, x_7, x_8, x_13); lean_dec(x_8); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_7); -lean_ctor_set(x_17, 1, x_15); -return x_17; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +return x_19; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; +uint8_t x_20; +lean_dec(x_8); lean_dec(x_7); -x_18 = lean_ctor_get(x_4, 0); -x_19 = lean_array_uget(x_18, x_6); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_2); -lean_inc(x_1); -lean_inc(x_3); -x_20 = l_Lean_Elab_Command_accLevelAtCtor(x_3, x_19, x_1, x_2, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -if (lean_obj_tag(x_20) == 0) +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_1); +x_20 = !lean_is_exclusive(x_10); +if (x_20 == 0) { -lean_object* x_21; size_t x_22; size_t x_23; lean_object* x_24; -x_21 = lean_ctor_get(x_20, 1); -lean_inc(x_21); -lean_dec(x_20); -x_22 = 1; -x_23 = lean_usize_add(x_6, x_22); +lean_object* x_21; lean_object* x_22; +x_21 = lean_ctor_get(x_10, 0); +lean_dec(x_21); +x_22 = lean_box(0); +lean_ctor_set(x_10, 0, x_22); +return x_10; +} +else +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_10, 1); +lean_inc(x_23); +lean_dec(x_10); x_24 = lean_box(0); -x_6 = x_23; -x_7 = x_24; -x_15 = x_21; -goto _start; +x_25 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_25, 0, x_24); +lean_ctor_set(x_25, 1, x_23); +return x_25; +} +} } else { uint8_t x_26; -lean_dec(x_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_26 = !lean_is_exclusive(x_20); +x_26 = !lean_is_exclusive(x_10); if (x_26 == 0) { -return x_20; +return x_10; } else { 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); +x_27 = lean_ctor_get(x_10, 0); +x_28 = lean_ctor_get(x_10, 1); lean_inc(x_28); lean_inc(x_27); -lean_dec(x_20); +lean_dec(x_10); x_29 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_29, 0, x_27); lean_ctor_set(x_29, 1, x_28); @@ -13877,2681 +14576,2779 @@ return x_29; } } } -} -LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___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, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__3___closed__1() { _start: { -lean_object* x_12; -x_12 = lean_apply_10(x_1, x_5, x_6, x_2, x_3, x_4, x_7, x_8, x_9, x_10, x_11); -return x_12; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("unexpected constructor resulting type", 37, 37); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__2___rarg(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) { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__3___closed__2() { _start: { -lean_object* x_12; lean_object* x_13; -x_12 = lean_alloc_closure((void*)(l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__2___rarg___lambda__1), 11, 4); -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_6); -x_13 = l___private_Lean_Meta_Basic_0__Lean_Meta_forallTelescopeReducingImp___rarg(x_1, x_12, x_3, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_13) == 0) -{ -uint8_t x_14; -x_14 = !lean_is_exclusive(x_13); -if (x_14 == 0) -{ -return x_13; +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__3___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } -else +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: { -lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = lean_ctor_get(x_13, 0); -x_16 = lean_ctor_get(x_13, 1); -lean_inc(x_16); -lean_inc(x_15); -lean_dec(x_13); -x_17 = lean_alloc_ctor(0, 2, 0); +lean_object* x_11; uint8_t x_12; +x_11 = l_Lean_Expr_getAppFn(x_3); +x_12 = lean_expr_eqv(x_11, x_1); +lean_dec(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; +x_13 = l_Lean_indentExpr(x_3); +x_14 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__3___closed__2; +x_15 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_13); +x_16 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +x_17 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_17, 0, x_15); lean_ctor_set(x_17, 1, x_16); -return x_17; -} -} -else -{ -uint8_t x_18; -x_18 = !lean_is_exclusive(x_13); -if (x_18 == 0) +x_18 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_17, 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); +x_19 = !lean_is_exclusive(x_18); +if (x_19 == 0) { -return x_13; +return x_18; } else { -lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_19 = lean_ctor_get(x_13, 0); -x_20 = lean_ctor_get(x_13, 1); +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_18, 0); +x_21 = lean_ctor_get(x_18, 1); +lean_inc(x_21); lean_inc(x_20); -lean_inc(x_19); -lean_dec(x_13); -x_21 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_21, 0, x_19); -lean_ctor_set(x_21, 1, x_20); -return x_21; -} -} +lean_dec(x_18); +x_22 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_22, 0, x_20); +lean_ctor_set(x_22, 1, x_21); +return x_22; } } -LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__2(lean_object* x_1) { -_start: +else { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__2___rarg___boxed), 11, 0); -return x_2; +lean_object* x_23; lean_object* x_24; +x_23 = lean_box(0); +x_24 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__2(x_3, x_23, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_24; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -uint8_t x_16; -x_16 = lean_usize_dec_lt(x_6, x_5); -if (x_16 == 0) +uint8_t x_14; uint8_t x_15; lean_object* x_16; +x_14 = 0; +x_15 = 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_16 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_14, x_15, 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_dec(x_14); -lean_dec(x_13); +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_16, 1); +lean_inc(x_17); +lean_dec(x_16); +x_18 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_1, x_7, x_8, x_9, x_10, x_11, x_12, 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); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +x_21 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs(x_2, x_3, x_19, x_9, x_10, x_11, x_12, x_20); +if (lean_obj_tag(x_21) == 0) +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; +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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__3___boxed), 10, 1); +lean_closure_set(x_24, 0, x_4); +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_22); +x_25 = l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___spec__1___rarg(x_22, x_24, x_15, x_7, x_8, x_9, x_10, x_11, x_12, x_23); +if (lean_obj_tag(x_25) == 0) +{ +lean_object* x_26; lean_object* x_27; +x_26 = lean_ctor_get(x_25, 1); +lean_inc(x_26); +lean_dec(x_25); +x_27 = lean_apply_8(x_5, x_22, x_7, x_8, x_9, x_10, x_11, x_12, x_26); +return x_27; +} +else +{ +uint8_t x_28; +lean_dec(x_22); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_3); -lean_dec(x_2); -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_7); -lean_ctor_set(x_17, 1, x_15); -return x_17; -} -else -{ -lean_object* x_18; lean_object* x_19; uint8_t x_20; lean_dec(x_7); -x_18 = lean_array_uget(x_4, x_6); -x_19 = lean_ctor_get(x_18, 2); -lean_inc(x_19); -x_20 = lean_name_eq(x_19, x_1); -lean_dec(x_19); -if (x_20 == 0) +lean_dec(x_5); +x_28 = !lean_is_exclusive(x_25); +if (x_28 == 0) { -size_t x_21; size_t x_22; -lean_dec(x_18); -x_21 = 1; -x_22 = lean_usize_add(x_6, x_21); -lean_inc(x_3); +return x_25; +} +else { -size_t _tmp_5 = x_22; -lean_object* _tmp_6 = x_3; -x_6 = _tmp_5; -x_7 = _tmp_6; +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_25, 0); +x_30 = lean_ctor_get(x_25, 1); +lean_inc(x_30); +lean_inc(x_29); +lean_dec(x_25); +x_31 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_31, 0, x_29); +lean_ctor_set(x_31, 1, x_30); +return x_31; +} } -goto _start; } else { -lean_object* x_24; uint8_t x_25; -lean_dec(x_3); -x_24 = lean_ctor_get(x_18, 0); -lean_inc(x_24); -lean_dec(x_18); -x_25 = !lean_is_exclusive(x_13); -if (x_25 == 0) -{ -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_13, 5); -x_27 = l_Lean_replaceRef(x_24, x_26); -lean_dec(x_26); -lean_dec(x_24); -lean_ctor_set(x_13, 5, x_27); -x_28 = lean_apply_8(x_2, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -if (lean_obj_tag(x_28) == 0) -{ -uint8_t x_29; -x_29 = !lean_is_exclusive(x_28); -if (x_29 == 0) +uint8_t x_32; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_4); +x_32 = !lean_is_exclusive(x_21); +if (x_32 == 0) { -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_30 = lean_ctor_get(x_28, 0); -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_28, 0, x_33); -return x_28; +return x_21; } else { -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_34 = lean_ctor_get(x_28, 0); -x_35 = lean_ctor_get(x_28, 1); -lean_inc(x_35); +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_21, 0); +x_34 = lean_ctor_get(x_21, 1); lean_inc(x_34); -lean_dec(x_28); -x_36 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_36, 0, x_34); -x_37 = lean_box(0); -x_38 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -x_39 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_39, 0, x_38); -lean_ctor_set(x_39, 1, x_35); -return x_39; +lean_inc(x_33); +lean_dec(x_21); +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +return x_35; +} } } else { -uint8_t x_40; -x_40 = !lean_is_exclusive(x_28); -if (x_40 == 0) +uint8_t x_36; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_36 = !lean_is_exclusive(x_16); +if (x_36 == 0) { -return x_28; +return x_16; } else { -lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_ctor_get(x_28, 0); -x_42 = lean_ctor_get(x_28, 1); -lean_inc(x_42); -lean_inc(x_41); -lean_dec(x_28); -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_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_16, 0); +x_38 = lean_ctor_get(x_16, 1); +lean_inc(x_38); +lean_inc(x_37); +lean_dec(x_16); +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 +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__1() { +_start: { -lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; uint8_t x_55; lean_object* x_56; uint8_t x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_44 = lean_ctor_get(x_13, 0); -x_45 = lean_ctor_get(x_13, 1); -x_46 = lean_ctor_get(x_13, 2); -x_47 = lean_ctor_get(x_13, 3); -x_48 = lean_ctor_get(x_13, 4); -x_49 = lean_ctor_get(x_13, 5); -x_50 = lean_ctor_get(x_13, 6); -x_51 = lean_ctor_get(x_13, 7); -x_52 = lean_ctor_get(x_13, 8); -x_53 = lean_ctor_get(x_13, 9); -x_54 = lean_ctor_get(x_13, 10); -x_55 = lean_ctor_get_uint8(x_13, sizeof(void*)*12); -x_56 = lean_ctor_get(x_13, 11); -x_57 = lean_ctor_get_uint8(x_13, sizeof(void*)*12 + 1); -lean_inc(x_56); -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_dec(x_13); -x_58 = l_Lean_replaceRef(x_24, x_49); -lean_dec(x_49); -lean_dec(x_24); -x_59 = lean_alloc_ctor(0, 12, 2); -lean_ctor_set(x_59, 0, x_44); -lean_ctor_set(x_59, 1, x_45); -lean_ctor_set(x_59, 2, x_46); -lean_ctor_set(x_59, 3, x_47); -lean_ctor_set(x_59, 4, x_48); -lean_ctor_set(x_59, 5, x_58); -lean_ctor_set(x_59, 6, x_50); -lean_ctor_set(x_59, 7, x_51); -lean_ctor_set(x_59, 8, x_52); -lean_ctor_set(x_59, 9, x_53); -lean_ctor_set(x_59, 10, x_54); -lean_ctor_set(x_59, 11, x_56); -lean_ctor_set_uint8(x_59, sizeof(void*)*12, x_55); -lean_ctor_set_uint8(x_59, sizeof(void*)*12 + 1, x_57); -x_60 = lean_apply_8(x_2, x_8, x_9, x_10, x_11, x_12, x_59, x_14, x_15); -if (lean_obj_tag(x_60) == 0) +lean_object* x_1; +x_1 = lean_mk_string_unchecked("constructor resulting type must be specified in inductive family declaration", 76, 76); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__2() { +_start: { -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_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); +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } -x_64 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_64, 0, x_61); -x_65 = lean_box(0); -x_66 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_66, 0, x_64); -lean_ctor_set(x_66, 1, x_65); -if (lean_is_scalar(x_63)) { - x_67 = lean_alloc_ctor(0, 2, 0); -} else { - x_67 = x_63; } -lean_ctor_set(x_67, 0, x_66); -lean_ctor_set(x_67, 1, x_62); -return x_67; +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("elabType ", 9, 9); +return x_1; } -else +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__4() { +_start: { -lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; -x_68 = lean_ctor_get(x_60, 0); -lean_inc(x_68); -x_69 = lean_ctor_get(x_60, 1); -lean_inc(x_69); -if (lean_is_exclusive(x_60)) { - lean_ctor_release(x_60, 0); - lean_ctor_release(x_60, 1); - x_70 = x_60; -} else { - lean_dec_ref(x_60); - x_70 = lean_box(0); +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } -if (lean_is_scalar(x_70)) { - x_71 = lean_alloc_ctor(1, 2, 0); -} else { - x_71 = x_70; } -lean_ctor_set(x_71, 0, x_68); -lean_ctor_set(x_71, 1, x_69); -return x_71; +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" : ", 3, 3); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__5; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__7() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" ", 1, 1); +return x_1; } } +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__7; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_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_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -uint8_t x_16; -x_16 = lean_usize_dec_lt(x_6, x_5); -if (x_16 == 0) +lean_object* x_14; +x_14 = lean_ctor_get(x_5, 4); +lean_inc(x_14); +if (lean_obj_tag(x_14) == 0) { -lean_object* x_17; -lean_dec(x_14); -lean_dec(x_13); +lean_dec(x_5); +lean_dec(x_1); +if (x_4 == 0) +{ +lean_object* x_15; lean_object* x_16; +x_15 = lean_box(0); +x_16 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__1(x_2, x_3, x_6, x_15, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_3); +return x_16; +} +else +{ +lean_object* x_17; lean_object* x_18; uint8_t x_19; +lean_dec(x_6); +lean_dec(x_3); +lean_dec(x_2); +x_17 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__2; +x_18 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_17, x_7, x_8, x_9, x_10, x_11, x_12, x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_3); -lean_dec(x_2); -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_7); -lean_ctor_set(x_17, 1, x_15); -return x_17; +x_19 = !lean_is_exclusive(x_18); +if (x_19 == 0) +{ +return x_18; } else { -lean_object* x_18; lean_object* x_19; size_t x_20; size_t x_21; lean_object* x_22; -lean_dec(x_7); -x_18 = lean_array_uget(x_4, x_6); -x_19 = lean_ctor_get(x_18, 8); -lean_inc(x_19); +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_18, 0); +x_21 = lean_ctor_get(x_18, 1); +lean_inc(x_21); +lean_inc(x_20); lean_dec(x_18); -x_20 = lean_array_size(x_19); -x_21 = 0; -lean_inc(x_14); -lean_inc(x_13); +x_22 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_22, 0, x_20); +lean_ctor_set(x_22, 1, x_21); +return x_22; +} +} +} +else +{ +lean_object* x_23; lean_object* x_24; +x_23 = lean_ctor_get(x_14, 0); +lean_inc(x_23); +lean_dec(x_14); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -lean_inc_n(x_3, 2); -lean_inc(x_2); -x_22 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__4(x_1, x_2, x_3, x_19, x_20, x_21, x_3, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -lean_dec(x_19); -if (lean_obj_tag(x_22) == 0) -{ -lean_object* x_23; lean_object* x_24; -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -lean_dec(x_23); +lean_inc(x_7); +x_24 = l_Lean_Elab_Term_elabType(x_23, x_7, x_8, x_9, x_10, x_11, x_12, x_13); if (lean_obj_tag(x_24) == 0) { -lean_object* x_25; size_t x_26; size_t x_27; -x_25 = lean_ctor_get(x_22, 1); +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_25 = lean_ctor_get(x_24, 0); lean_inc(x_25); -lean_dec(x_22); -x_26 = 1; -x_27 = lean_usize_add(x_6, x_26); -lean_inc(x_3); +x_26 = lean_ctor_get(x_24, 1); +lean_inc(x_26); +lean_dec(x_24); +x_27 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__3; +x_28 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_27, x_7, x_8, x_9, x_10, x_11, x_12, x_26); +x_29 = lean_ctor_get(x_28, 0); +lean_inc(x_29); +x_30 = lean_unbox(x_29); +lean_dec(x_29); +if (x_30 == 0) { -size_t _tmp_5 = x_27; -lean_object* _tmp_6 = x_3; -lean_object* _tmp_14 = x_25; -x_6 = _tmp_5; -x_7 = _tmp_6; -x_15 = _tmp_14; +lean_object* x_31; lean_object* x_32; lean_object* x_33; +lean_dec(x_5); +x_31 = lean_ctor_get(x_28, 1); +lean_inc(x_31); +lean_dec(x_28); +x_32 = lean_box(0); +x_33 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__4(x_25, x_1, x_3, x_2, x_6, x_32, x_7, x_8, x_9, x_10, x_11, x_12, x_31); +return x_33; } -goto _start; +else +{ +uint8_t x_34; +x_34 = !lean_is_exclusive(x_28); +if (x_34 == 0) +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_35 = lean_ctor_get(x_28, 1); +x_36 = lean_ctor_get(x_28, 0); +lean_dec(x_36); +x_37 = lean_ctor_get(x_5, 2); +lean_inc(x_37); +lean_dec(x_5); +x_38 = l_Lean_MessageData_ofName(x_37); +x_39 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__4; +lean_ctor_set_tag(x_28, 7); +lean_ctor_set(x_28, 1, x_38); +lean_ctor_set(x_28, 0, x_39); +x_40 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__6; +x_41 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_41, 0, x_28); +lean_ctor_set(x_41, 1, x_40); +lean_inc(x_25); +x_42 = l_Lean_MessageData_ofExpr(x_25); +x_43 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_43, 0, x_41); +lean_ctor_set(x_43, 1, x_42); +x_44 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__8; +x_45 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_45, 0, x_43); +lean_ctor_set(x_45, 1, x_44); +x_46 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_27, x_45, x_7, x_8, x_9, x_10, x_11, x_12, x_35); +x_47 = lean_ctor_get(x_46, 0); +lean_inc(x_47); +x_48 = lean_ctor_get(x_46, 1); +lean_inc(x_48); +lean_dec(x_46); +x_49 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__4(x_25, x_1, x_3, x_2, x_6, x_47, x_7, x_8, x_9, x_10, x_11, x_12, x_48); +lean_dec(x_47); +return x_49; } else { -uint8_t x_29; -lean_dec(x_14); -lean_dec(x_13); +lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; +x_50 = lean_ctor_get(x_28, 1); +lean_inc(x_50); +lean_dec(x_28); +x_51 = lean_ctor_get(x_5, 2); +lean_inc(x_51); +lean_dec(x_5); +x_52 = l_Lean_MessageData_ofName(x_51); +x_53 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__4; +x_54 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_54, 0, x_53); +lean_ctor_set(x_54, 1, x_52); +x_55 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__6; +x_56 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_56, 0, x_54); +lean_ctor_set(x_56, 1, x_55); +lean_inc(x_25); +x_57 = l_Lean_MessageData_ofExpr(x_25); +x_58 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_58, 0, x_56); +lean_ctor_set(x_58, 1, x_57); +x_59 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__8; +x_60 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_60, 0, x_58); +lean_ctor_set(x_60, 1, x_59); +x_61 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_27, x_60, x_7, x_8, x_9, x_10, x_11, x_12, x_50); +x_62 = lean_ctor_get(x_61, 0); +lean_inc(x_62); +x_63 = lean_ctor_get(x_61, 1); +lean_inc(x_63); +lean_dec(x_61); +x_64 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__4(x_25, x_1, x_3, x_2, x_6, x_62, x_7, x_8, x_9, x_10, x_11, x_12, x_63); +lean_dec(x_62); +return x_64; +} +} +} +else +{ +uint8_t x_65; lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); lean_dec(x_3); lean_dec(x_2); -x_29 = !lean_is_exclusive(x_22); -if (x_29 == 0) -{ -lean_object* x_30; uint8_t x_31; -x_30 = lean_ctor_get(x_22, 0); -lean_dec(x_30); -x_31 = !lean_is_exclusive(x_24); -if (x_31 == 0) +lean_dec(x_1); +x_65 = !lean_is_exclusive(x_24); +if (x_65 == 0) { -lean_object* x_32; lean_object* x_33; -x_32 = lean_box(0); -x_33 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_33, 0, x_24); -lean_ctor_set(x_33, 1, x_32); -lean_ctor_set(x_22, 0, x_33); -return x_22; +return x_24; } else { -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_34 = lean_ctor_get(x_24, 0); -lean_inc(x_34); +lean_object* x_66; lean_object* x_67; lean_object* x_68; +x_66 = lean_ctor_get(x_24, 0); +x_67 = lean_ctor_get(x_24, 1); +lean_inc(x_67); +lean_inc(x_66); lean_dec(x_24); -x_35 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_35, 0, x_34); -x_36 = lean_box(0); -x_37 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -lean_ctor_set(x_22, 0, x_37); -return x_22; +x_68 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_68, 0, x_66); +lean_ctor_set(x_68, 1, x_67); +return x_68; } } -else -{ -lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_38 = lean_ctor_get(x_22, 1); -lean_inc(x_38); -lean_dec(x_22); -x_39 = lean_ctor_get(x_24, 0); -lean_inc(x_39); -if (lean_is_exclusive(x_24)) { - lean_ctor_release(x_24, 0); - x_40 = x_24; -} else { - lean_dec_ref(x_24); - 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_box(0); -x_43 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_43, 0, x_41); -lean_ctor_set(x_43, 1, x_42); -x_44 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_44, 0, x_43); -lean_ctor_set(x_44, 1, x_38); -return x_44; } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +x_12 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___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_2); +return x_12; } } -else +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: { -uint8_t x_45; -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_3); +lean_object* x_10; +x_10 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_4); lean_dec(x_2); -x_45 = !lean_is_exclusive(x_22); -if (x_45 == 0) -{ -return x_22; +return x_10; } -else -{ -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; } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_5); +lean_dec(x_2); +lean_dec(x_1); +return x_11; } } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; +x_14 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_6); +return x_14; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_withCtorRef___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___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_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -lean_object* x_11; -x_11 = lean_apply_8(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_11; +uint8_t x_14; lean_object* x_15; +x_14 = lean_unbox(x_4); +lean_dec(x_4); +x_15 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType(x_1, x_2, x_3, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +return x_15; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_withCtorRef___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___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 uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__1(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4) { _start: { -size_t x_12; size_t x_13; lean_object* x_14; lean_object* x_15; -x_12 = lean_array_size(x_1); -x_13 = 0; -x_14 = l_Lean_Elab_Command_withCtorRef___rarg___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_4); -lean_inc(x_3); -x_15 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__5(x_2, x_3, x_14, x_1, x_12, x_13, x_14, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_15) == 0) +uint8_t x_5; +x_5 = lean_usize_dec_eq(x_3, x_4); +if (x_5 == 0) { -lean_object* x_16; lean_object* x_17; -x_16 = lean_ctor_get(x_15, 0); -lean_inc(x_16); -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -lean_dec(x_16); -if (lean_obj_tag(x_17) == 0) +lean_object* x_6; uint8_t x_7; +x_6 = lean_array_uget(x_2, x_3); +x_7 = l_Lean_Expr_isMVar(x_6); +if (x_7 == 0) { -lean_object* x_18; lean_object* x_19; -x_18 = lean_ctor_get(x_15, 1); -lean_inc(x_18); -lean_dec(x_15); -x_19 = lean_apply_8(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_18); -return x_19; +size_t x_8; size_t x_9; +lean_dec(x_6); +x_8 = 1; +x_9 = lean_usize_add(x_3, x_8); +x_3 = x_9; +goto _start; } else { -uint8_t x_20; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); +lean_object* x_11; uint8_t x_12; +x_11 = l_Lean_Expr_mvarId_x21(x_6); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_20 = !lean_is_exclusive(x_15); -if (x_20 == 0) +x_12 = lean_name_eq(x_11, x_1); +lean_dec(x_11); +if (x_12 == 0) { -lean_object* x_21; lean_object* x_22; -x_21 = lean_ctor_get(x_15, 0); -lean_dec(x_21); -x_22 = lean_ctor_get(x_17, 0); -lean_inc(x_22); -lean_dec(x_17); -lean_ctor_set(x_15, 0, x_22); -return x_15; +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 { -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_15, 1); -lean_inc(x_23); -lean_dec(x_15); -x_24 = lean_ctor_get(x_17, 0); -lean_inc(x_24); -lean_dec(x_17); -x_25 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_25, 0, x_24); -lean_ctor_set(x_25, 1, x_23); -return x_25; +uint8_t x_16; +x_16 = 1; +return x_16; } } } else { -uint8_t x_26; -lean_dec(x_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 = !lean_is_exclusive(x_15); -if (x_26 == 0) +uint8_t x_17; +x_17 = 0; +return x_17; +} +} +} +LEAN_EXPORT uint8_t l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__1(lean_object* x_1, lean_object* x_2) { +_start: { -return x_15; +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 { -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_15, 0); -x_28 = lean_ctor_get(x_15, 1); -lean_inc(x_28); -lean_inc(x_27); -lean_dec(x_15); -x_29 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_29, 0, x_27); -lean_ctor_set(x_29, 1, x_28); -return x_29; +size_t x_7; size_t x_8; uint8_t x_9; +x_7 = 0; +x_8 = lean_usize_of_nat(x_3); +lean_dec(x_3); +x_9 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__1(x_2, x_1, x_7, x_8); +return x_9; +} } } +LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_1, 2); +lean_inc(x_11); +x_12 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_11); +lean_ctor_set(x_12, 1, x_2); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_10); +return x_13; } } -LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___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, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { -lean_object* x_15; lean_object* x_16; lean_object* x_17; size_t x_18; lean_object* x_19; size_t x_20; lean_object* x_21; lean_object* x_22; -x_15 = lean_array_get_size(x_5); -x_16 = l_Array_toSubarray___rarg(x_5, x_1, x_15); -x_17 = lean_ctor_get(x_16, 2); -lean_inc(x_17); -x_18 = lean_usize_of_nat(x_17); -lean_dec(x_17); -x_19 = lean_ctor_get(x_16, 1); -lean_inc(x_19); -x_20 = lean_usize_of_nat(x_19); +lean_object* x_15; uint8_t x_16; uint8_t x_17; uint8_t x_18; lean_object* x_19; +x_15 = l_Array_append___rarg(x_1, x_2); +x_16 = 0; +x_17 = 1; +x_18 = 1; +x_19 = l_Lean_Meta_mkForallFVars(x_15, x_3, x_16, x_17, x_18, x_10, x_11, x_12, x_13, x_14); +if (lean_obj_tag(x_19) == 0) +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_19, 1); +lean_inc(x_21); lean_dec(x_19); -x_21 = lean_box(0); -x_22 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__1(x_2, x_3, x_4, x_16, x_18, x_20, x_21, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -lean_dec(x_16); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +x_22 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs(x_20, x_10, x_11, x_12, x_13, x_21); if (lean_obj_tag(x_22) == 0) { -uint8_t x_23; -x_23 = !lean_is_exclusive(x_22); -if (x_23 == 0) +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +lean_dec(x_22); +x_25 = l_Lean_Meta_mkForallFVars(x_4, x_23, x_16, x_17, x_18, x_10, x_11, x_12, x_13, x_24); +if (lean_obj_tag(x_25) == 0) { -lean_object* x_24; -x_24 = lean_ctor_get(x_22, 0); -lean_dec(x_24); -lean_ctor_set(x_22, 0, x_21); -return x_22; -} -else +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; +x_26 = lean_ctor_get(x_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_5); +x_28 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_5, x_8, x_9, x_10, x_11, x_12, x_13, x_27); +x_29 = lean_ctor_get(x_28, 0); +lean_inc(x_29); +x_30 = lean_unbox(x_29); +lean_dec(x_29); +if (x_30 == 0) { -lean_object* x_25; lean_object* x_26; -x_25 = lean_ctor_get(x_22, 1); -lean_inc(x_25); -lean_dec(x_22); -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_21); -lean_ctor_set(x_26, 1, x_25); -return x_26; -} +lean_object* x_31; lean_object* x_32; lean_object* x_33; +lean_dec(x_5); +x_31 = lean_ctor_get(x_28, 1); +lean_inc(x_31); +lean_dec(x_28); +x_32 = lean_box(0); +x_33 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__2(x_6, x_26, x_32, x_8, x_9, x_10, x_11, x_12, x_13, x_31); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_6); +return x_33; } else { -uint8_t x_27; -x_27 = !lean_is_exclusive(x_22); -if (x_27 == 0) +uint8_t x_34; +x_34 = !lean_is_exclusive(x_28); +if (x_34 == 0) { -return x_22; +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_35 = lean_ctor_get(x_28, 1); +x_36 = lean_ctor_get(x_28, 0); +lean_dec(x_36); +x_37 = lean_ctor_get(x_6, 2); +lean_inc(x_37); +x_38 = l_Lean_MessageData_ofName(x_37); +x_39 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +lean_ctor_set_tag(x_28, 7); +lean_ctor_set(x_28, 1, x_38); +lean_ctor_set(x_28, 0, x_39); +x_40 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__6; +x_41 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_41, 0, x_28); +lean_ctor_set(x_41, 1, x_40); +lean_inc(x_26); +x_42 = l_Lean_MessageData_ofExpr(x_26); +x_43 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_43, 0, x_41); +lean_ctor_set(x_43, 1, x_42); +x_44 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_44, 0, x_43); +lean_ctor_set(x_44, 1, x_39); +x_45 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_5, x_44, x_8, x_9, x_10, x_11, x_12, x_13, x_35); +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_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__2(x_6, x_26, x_46, x_8, x_9, x_10, x_11, x_12, x_13, x_47); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_46); +lean_dec(x_6); +return x_48; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_28 = lean_ctor_get(x_22, 0); -x_29 = lean_ctor_get(x_22, 1); -lean_inc(x_29); -lean_inc(x_28); -lean_dec(x_22); -x_30 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_30, 0, x_28); -lean_ctor_set(x_30, 1, x_29); -return x_30; -} +lean_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_49 = lean_ctor_get(x_28, 1); +lean_inc(x_49); +lean_dec(x_28); +x_50 = lean_ctor_get(x_6, 2); +lean_inc(x_50); +x_51 = l_Lean_MessageData_ofName(x_50); +x_52 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +x_53 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_53, 0, x_52); +lean_ctor_set(x_53, 1, x_51); +x_54 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__6; +x_55 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_55, 0, x_53); +lean_ctor_set(x_55, 1, x_54); +lean_inc(x_26); +x_56 = l_Lean_MessageData_ofExpr(x_26); +x_57 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_57, 0, x_55); +lean_ctor_set(x_57, 1, x_56); +x_58 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_58, 0, x_57); +lean_ctor_set(x_58, 1, x_52); +x_59 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_5, x_58, x_8, x_9, x_10, x_11, x_12, x_13, x_49); +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_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__2(x_6, x_26, x_60, x_8, x_9, x_10, x_11, x_12, x_13, x_61); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_60); +lean_dec(x_6); +return x_62; } } } -LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { -_start: -{ -if (lean_obj_tag(x_5) == 0) +else { -lean_object* x_14; lean_object* x_15; +uint8_t x_63; +lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); lean_dec(x_6); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_14 = lean_box(0); -x_15 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_15, 0, x_14); -lean_ctor_set(x_15, 1, x_13); -return x_15; +lean_dec(x_5); +x_63 = !lean_is_exclusive(x_25); +if (x_63 == 0) +{ +return x_25; } else { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_16 = lean_ctor_get(x_5, 0); -lean_inc(x_16); -x_17 = lean_ctor_get(x_5, 1); -lean_inc(x_17); -lean_dec(x_5); -x_18 = lean_ctor_get(x_16, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_16, 1); -lean_inc(x_19); -lean_inc(x_3); -lean_inc(x_2); -lean_inc(x_4); -x_20 = lean_alloc_closure((void*)(l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__6___lambda__1___boxed), 14, 4); -lean_closure_set(x_20, 0, x_4); -lean_closure_set(x_20, 1, x_2); -lean_closure_set(x_20, 2, x_3); -lean_closure_set(x_20, 3, x_16); -x_21 = 0; -x_22 = lean_box(x_21); -x_23 = lean_alloc_closure((void*)(l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__2___rarg___boxed), 11, 3); -lean_closure_set(x_23, 0, x_19); -lean_closure_set(x_23, 1, x_20); -lean_closure_set(x_23, 2, x_22); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -x_24 = l_Lean_Elab_Command_withCtorRef___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__3(x_1, x_18, x_23, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_18); -if (lean_obj_tag(x_24) == 0) -{ -lean_object* x_25; -x_25 = lean_ctor_get(x_24, 1); -lean_inc(x_25); -lean_dec(x_24); -x_5 = x_17; -x_13 = x_25; -goto _start; +lean_object* x_64; lean_object* x_65; lean_object* x_66; +x_64 = lean_ctor_get(x_25, 0); +x_65 = lean_ctor_get(x_25, 1); +lean_inc(x_65); +lean_inc(x_64); +lean_dec(x_25); +x_66 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_66, 0, x_64); +lean_ctor_set(x_66, 1, x_65); +return x_66; +} +} } else { -uint8_t x_27; -lean_dec(x_17); +uint8_t x_67; +lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_27 = !lean_is_exclusive(x_24); -if (x_27 == 0) +x_67 = !lean_is_exclusive(x_22); +if (x_67 == 0) { -return x_24; +return x_22; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_28 = lean_ctor_get(x_24, 0); -x_29 = lean_ctor_get(x_24, 1); -lean_inc(x_29); -lean_inc(x_28); -lean_dec(x_24); -x_30 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_30, 0, x_28); -lean_ctor_set(x_30, 1, x_29); -return x_30; -} -} -} -} +lean_object* x_68; lean_object* x_69; lean_object* x_70; +x_68 = lean_ctor_get(x_22, 0); +x_69 = lean_ctor_get(x_22, 1); +lean_inc(x_69); +lean_inc(x_68); +lean_dec(x_22); +x_70 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_70, 0, x_68); +lean_ctor_set(x_70, 1, x_69); +return x_70; } -LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { -_start: -{ -if (lean_obj_tag(x_5) == 0) -{ -lean_object* x_14; lean_object* x_15; -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_14 = lean_box(0); -x_15 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_15, 0, x_14); -lean_ctor_set(x_15, 1, x_13); -return x_15; } -else -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_16 = lean_ctor_get(x_5, 0); -lean_inc(x_16); -x_17 = lean_ctor_get(x_5, 1); -lean_inc(x_17); -lean_dec(x_5); -x_18 = lean_ctor_get(x_16, 2); -lean_inc(x_18); -lean_dec(x_16); -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_4); -lean_inc(x_3); -lean_inc(x_2); -x_19 = l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__6(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); -if (lean_obj_tag(x_19) == 0) -{ -lean_object* x_20; -x_20 = lean_ctor_get(x_19, 1); -lean_inc(x_20); -lean_dec(x_19); -x_5 = x_17; -x_13 = x_20; -goto _start; } else { -uint8_t x_22; -lean_dec(x_17); +uint8_t x_71; +lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_22 = !lean_is_exclusive(x_19); -if (x_22 == 0) +x_71 = !lean_is_exclusive(x_19); +if (x_71 == 0) { return x_19; } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_19, 0); -x_24 = lean_ctor_get(x_19, 1); -lean_inc(x_24); -lean_inc(x_23); +lean_object* x_72; lean_object* x_73; lean_object* x_74; +x_72 = lean_ctor_get(x_19, 0); +x_73 = lean_ctor_get(x_19, 1); +lean_inc(x_73); +lean_inc(x_72); lean_dec(x_19); -x_25 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_25, 0, x_23); -lean_ctor_set(x_25, 1, x_24); -return x_25; -} +x_74 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_74, 0, x_72); +lean_ctor_set(x_74, 1, x_73); +return x_74; } } } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +static lean_object* _init_l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__4___closed__1() { _start: { -lean_object* x_14; -x_14 = l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___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); -return x_14; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("extraCtorParams: ", 17, 17); +return x_1; } } -LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +static lean_object* _init_l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__4___closed__2() { _start: { -size_t x_16; size_t x_17; lean_object* x_18; -x_16 = lean_unbox_usize(x_5); -lean_dec(x_5); -x_17 = lean_unbox_usize(x_6); -lean_dec(x_6); -x_18 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__1(x_1, x_2, x_3, x_4, x_16, x_17, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -lean_dec(x_4); -return x_18; +lean_object* x_1; lean_object* x_2; +x_1 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__4___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__2___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___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_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -uint8_t x_12; lean_object* x_13; -x_12 = lean_unbox(x_3); -lean_dec(x_3); -x_13 = l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__2___rarg(x_1, x_2, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -return x_13; -} -} -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { -_start: +uint8_t x_12; uint8_t x_13; lean_object* x_14; +x_12 = 1; +x_13 = 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_14 = l_Lean_Elab_Term_synthesizeSyntheticMVars(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) { -size_t x_16; size_t x_17; lean_object* x_18; -x_16 = lean_unbox_usize(x_5); -lean_dec(x_5); -x_17 = lean_unbox_usize(x_6); +lean_object* x_15; lean_object* x_16; +x_15 = lean_ctor_get(x_14, 1); +lean_inc(x_15); +lean_dec(x_14); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_5); +x_16 = l_Lean_Elab_Term_addAutoBoundImplicits(x_1, x_5, x_6, x_7, x_8, x_9, x_10, x_15); +if (lean_obj_tag(x_16) == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +lean_inc(x_17); +x_19 = lean_alloc_closure((void*)(l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__1___boxed), 2, 1); +lean_closure_set(x_19, 0, x_17); +lean_inc(x_4); +x_20 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_18); +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +x_23 = lean_box(0); +x_24 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__8___closed__1; +x_25 = l_Lean_Elab_Term_collectUnassignedMVars(x_21, x_24, x_19, x_5, x_6, x_7, x_8, x_9, x_10, x_22); +x_26 = !lean_is_exclusive(x_25); +if (x_26 == 0) +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; +x_27 = lean_ctor_get(x_25, 0); +x_28 = lean_ctor_get(x_25, 1); +x_29 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__3; +x_30 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_29, x_5, x_6, x_7, x_8, x_9, x_10, x_28); +x_31 = lean_ctor_get(x_30, 0); +lean_inc(x_31); +x_32 = lean_unbox(x_31); +lean_dec(x_31); +if (x_32 == 0) +{ +lean_object* x_33; lean_object* x_34; lean_object* x_35; +lean_free_object(x_25); +x_33 = lean_ctor_get(x_30, 1); +lean_inc(x_33); +lean_dec(x_30); +x_34 = lean_box(0); +x_35 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__3(x_27, x_17, x_4, x_2, x_29, x_3, x_34, x_5, x_6, x_7, x_8, x_9, x_10, x_33); lean_dec(x_6); -x_18 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__4(x_1, x_2, x_3, x_4, x_16, x_17, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -lean_dec(x_4); -lean_dec(x_1); -return x_18; -} +lean_dec(x_5); +lean_dec(x_17); +return x_35; } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { -_start: +else { -size_t x_16; size_t x_17; lean_object* x_18; -x_16 = lean_unbox_usize(x_5); -lean_dec(x_5); -x_17 = lean_unbox_usize(x_6); +uint8_t x_36; +x_36 = !lean_is_exclusive(x_30); +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; lean_object* x_46; lean_object* x_47; +x_37 = lean_ctor_get(x_30, 1); +x_38 = lean_ctor_get(x_30, 0); +lean_dec(x_38); +lean_inc(x_27); +x_39 = lean_array_to_list(x_27); +x_40 = l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(x_39, x_23); +x_41 = l_Lean_MessageData_ofList(x_40); +x_42 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__4___closed__2; +lean_ctor_set_tag(x_30, 7); +lean_ctor_set(x_30, 1, x_41); +lean_ctor_set(x_30, 0, x_42); +x_43 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +lean_ctor_set_tag(x_25, 7); +lean_ctor_set(x_25, 1, x_43); +lean_ctor_set(x_25, 0, x_30); +x_44 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_29, x_25, x_5, x_6, x_7, x_8, x_9, x_10, x_37); +x_45 = lean_ctor_get(x_44, 0); +lean_inc(x_45); +x_46 = lean_ctor_get(x_44, 1); +lean_inc(x_46); +lean_dec(x_44); +x_47 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__3(x_27, x_17, x_4, x_2, x_29, x_3, x_45, x_5, x_6, x_7, x_8, x_9, x_10, x_46); lean_dec(x_6); -x_18 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__5(x_1, x_2, x_3, x_4, x_16, x_17, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -lean_dec(x_4); -lean_dec(x_1); -return x_18; -} +lean_dec(x_5); +lean_dec(x_45); +lean_dec(x_17); +return x_47; } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_withCtorRef___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__3___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: +else { -lean_object* x_11; -x_11 = l_Lean_Elab_Command_withCtorRef___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__3___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_2); -return x_11; -} +lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; +x_48 = lean_ctor_get(x_30, 1); +lean_inc(x_48); +lean_dec(x_30); +lean_inc(x_27); +x_49 = lean_array_to_list(x_27); +x_50 = l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(x_49, x_23); +x_51 = l_Lean_MessageData_ofList(x_50); +x_52 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__4___closed__2; +x_53 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_53, 0, x_52); +lean_ctor_set(x_53, 1, x_51); +x_54 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +lean_ctor_set_tag(x_25, 7); +lean_ctor_set(x_25, 1, x_54); +lean_ctor_set(x_25, 0, x_53); +x_55 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_29, x_25, x_5, x_6, x_7, x_8, x_9, x_10, x_48); +x_56 = lean_ctor_get(x_55, 0); +lean_inc(x_56); +x_57 = lean_ctor_get(x_55, 1); +lean_inc(x_57); +lean_dec(x_55); +x_58 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__3(x_27, x_17, x_4, x_2, x_29, x_3, x_56, x_5, x_6, x_7, x_8, x_9, x_10, x_57); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_56); +lean_dec(x_17); +return x_58; } -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* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, 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_Command_withCtorRef___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_2); -lean_dec(x_1); -return x_12; } } -LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___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_object* x_12, lean_object* x_13, lean_object* x_14) { -_start: +else { -lean_object* x_15; -x_15 = l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__6___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_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_ctor_get(x_25, 0); +x_60 = lean_ctor_get(x_25, 1); +lean_inc(x_60); +lean_inc(x_59); +lean_dec(x_25); +x_61 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__3; +x_62 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_61, x_5, x_6, x_7, x_8, x_9, x_10, x_60); +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) +{ +lean_object* x_65; lean_object* x_66; lean_object* x_67; +x_65 = lean_ctor_get(x_62, 1); +lean_inc(x_65); +lean_dec(x_62); +x_66 = lean_box(0); +x_67 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__3(x_59, x_17, x_4, x_2, x_61, x_3, x_66, x_5, x_6, x_7, x_8, x_9, x_10, x_65); lean_dec(x_6); -return x_15; -} +lean_dec(x_5); +lean_dec(x_17); +return x_67; } -LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_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, lean_object* x_11, lean_object* x_12, lean_object* x_13) { -_start: +else { -lean_object* x_14; -x_14 = l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_1); -return x_14; -} +lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; +x_68 = lean_ctor_get(x_62, 1); +lean_inc(x_68); +if (lean_is_exclusive(x_62)) { + lean_ctor_release(x_62, 0); + lean_ctor_release(x_62, 1); + x_69 = x_62; +} else { + lean_dec_ref(x_62); + x_69 = lean_box(0); } -LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { -_start: -{ -lean_object* x_14; -x_14 = l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___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_1); -return x_14; +lean_inc(x_59); +x_70 = lean_array_to_list(x_59); +x_71 = l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(x_70, x_23); +x_72 = l_Lean_MessageData_ofList(x_71); +x_73 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__4___closed__2; +if (lean_is_scalar(x_69)) { + x_74 = lean_alloc_ctor(7, 2, 0); +} else { + x_74 = x_69; + lean_ctor_set_tag(x_74, 7); } +lean_ctor_set(x_74, 0, x_73); +lean_ctor_set(x_74, 1, x_72); +x_75 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +x_76 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_76, 0, x_74); +lean_ctor_set(x_76, 1, x_75); +x_77 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_61, x_76, x_5, x_6, x_7, x_8, x_9, x_10, x_68); +x_78 = lean_ctor_get(x_77, 0); +lean_inc(x_78); +x_79 = lean_ctor_get(x_77, 1); +lean_inc(x_79); +lean_dec(x_77); +x_80 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__3(x_59, x_17, x_4, x_2, x_61, x_3, x_78, x_5, x_6, x_7, x_8, x_9, x_10, x_79); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_78); +lean_dec(x_17); +return x_80; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { -_start: -{ -lean_object* x_14; -x_14 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_1); -return x_14; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_13 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__3___closed__1; -x_14 = lean_st_mk_ref(x_13, x_12); -x_15 = lean_ctor_get(x_14, 0); -lean_inc(x_15); -x_16 = lean_ctor_get(x_14, 1); -lean_inc(x_16); -lean_dec(x_14); -lean_inc(x_15); -x_17 = l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__7(x_1, x_2, x_3, x_4, x_5, x_15, x_6, x_7, x_8, x_9, x_10, x_11, x_16); -if (lean_obj_tag(x_17) == 0) +else { -lean_object* x_18; lean_object* x_19; uint8_t x_20; -x_18 = lean_ctor_get(x_17, 1); -lean_inc(x_18); -lean_dec(x_17); -x_19 = lean_st_ref_get(x_15, x_18); -lean_dec(x_15); -x_20 = !lean_is_exclusive(x_19); -if (x_20 == 0) +uint8_t x_81; +lean_dec(x_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_81 = !lean_is_exclusive(x_16); +if (x_81 == 0) { -return x_19; +return x_16; } else { -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_19, 0); -x_22 = lean_ctor_get(x_19, 1); -lean_inc(x_22); -lean_inc(x_21); -lean_dec(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); -return x_23; +lean_object* x_82; lean_object* x_83; lean_object* x_84; +x_82 = lean_ctor_get(x_16, 0); +x_83 = lean_ctor_get(x_16, 1); +lean_inc(x_83); +lean_inc(x_82); +lean_dec(x_16); +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_24; -lean_dec(x_15); -x_24 = !lean_is_exclusive(x_17); -if (x_24 == 0) +uint8_t x_85; +lean_dec(x_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_85 = !lean_is_exclusive(x_14); +if (x_85 == 0) { -return x_17; +return x_14; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_17, 0); -x_26 = lean_ctor_get(x_17, 1); -lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_17); -x_27 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_26); -return x_27; +lean_object* x_86; lean_object* x_87; lean_object* x_88; +x_86 = lean_ctor_get(x_14, 0); +x_87 = lean_ctor_get(x_14, 1); +lean_inc(x_87); +lean_inc(x_86); +lean_dec(x_14); +x_88 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_88, 0, x_86); +lean_ctor_set(x_88, 1, x_87); +return x_88; } } } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_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_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__5(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) { _start: { -lean_object* x_13; -x_13 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_1); -return x_13; -} +lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_14 = lean_ctor_get(x_1, 0); +lean_inc(x_14); +lean_inc(x_1); +lean_inc(x_2); +x_15 = lean_alloc_closure((void*)(l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__4___boxed), 11, 3); +lean_closure_set(x_15, 0, x_6); +lean_closure_set(x_15, 1, x_2); +lean_closure_set(x_15, 2, x_1); +x_16 = !lean_is_exclusive(x_11); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_11, 5); +x_18 = l_Lean_replaceRef(x_14, x_17); +lean_dec(x_17); +lean_dec(x_14); +lean_ctor_set(x_11, 5, x_18); +x_19 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType(x_3, x_4, x_2, x_5, x_1, x_15, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +return x_19; } -LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___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) { -_start: +else { -lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_9 = lean_array_get_size(x_2); -x_10 = lean_nat_sub(x_9, x_1); -lean_dec(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_8); -return x_11; -} -} -static lean_object* _init_l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__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; -} +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; uint8_t x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_20 = lean_ctor_get(x_11, 0); +x_21 = lean_ctor_get(x_11, 1); +x_22 = lean_ctor_get(x_11, 2); +x_23 = lean_ctor_get(x_11, 3); +x_24 = lean_ctor_get(x_11, 4); +x_25 = lean_ctor_get(x_11, 5); +x_26 = lean_ctor_get(x_11, 6); +x_27 = lean_ctor_get(x_11, 7); +x_28 = lean_ctor_get(x_11, 8); +x_29 = lean_ctor_get(x_11, 9); +x_30 = lean_ctor_get(x_11, 10); +x_31 = lean_ctor_get_uint8(x_11, sizeof(void*)*12); +x_32 = lean_ctor_get(x_11, 11); +x_33 = lean_ctor_get_uint8(x_11, sizeof(void*)*12 + 1); +lean_inc(x_32); +lean_inc(x_30); +lean_inc(x_29); +lean_inc(x_28); +lean_inc(x_27); +lean_inc(x_26); +lean_inc(x_25); +lean_inc(x_24); +lean_inc(x_23); +lean_inc(x_22); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_11); +x_34 = l_Lean_replaceRef(x_14, x_25); +lean_dec(x_25); +lean_dec(x_14); +x_35 = lean_alloc_ctor(0, 12, 2); +lean_ctor_set(x_35, 0, x_20); +lean_ctor_set(x_35, 1, x_21); +lean_ctor_set(x_35, 2, x_22); +lean_ctor_set(x_35, 3, x_23); +lean_ctor_set(x_35, 4, x_24); +lean_ctor_set(x_35, 5, x_34); +lean_ctor_set(x_35, 6, x_26); +lean_ctor_set(x_35, 7, x_27); +lean_ctor_set(x_35, 8, x_28); +lean_ctor_set(x_35, 9, x_29); +lean_ctor_set(x_35, 10, x_30); +lean_ctor_set(x_35, 11, x_32); +lean_ctor_set_uint8(x_35, sizeof(void*)*12, x_31); +lean_ctor_set_uint8(x_35, sizeof(void*)*12 + 1, x_33); +x_36 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType(x_3, x_4, x_2, x_5, x_1, x_15, x_7, x_8, x_9, x_10, x_35, x_12, x_13); +return x_36; } -static lean_object* _init_l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__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_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__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; } } -LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -if (lean_obj_tag(x_3) == 0) +if (lean_obj_tag(x_5) == 0) { -lean_object* x_10; +lean_object* x_14; lean_object* x_15; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_4); -lean_ctor_set(x_10, 1, x_9); -return x_10; +x_14 = l_List_reverse___rarg(x_6); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_13); +return x_15; } else { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; lean_object* x_16; -lean_dec(x_4); -x_11 = lean_ctor_get(x_3, 0); -lean_inc(x_11); -x_12 = lean_ctor_get(x_3, 1); -lean_inc(x_12); -lean_dec(x_3); -x_13 = lean_ctor_get(x_11, 1); -lean_inc(x_13); -lean_dec(x_11); +uint8_t x_16; +x_16 = !lean_is_exclusive(x_5); +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; +x_17 = lean_ctor_get(x_5, 0); +x_18 = lean_ctor_get(x_5, 1); +x_19 = lean_ctor_get(x_17, 3); +lean_inc(x_19); +x_20 = l_Lean_Syntax_getArgs(x_19); +lean_dec(x_19); +x_21 = lean_box(x_4); +lean_inc(x_2); lean_inc(x_1); -x_14 = lean_alloc_closure((void*)(l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__1___lambda__1___boxed), 8, 1); -lean_closure_set(x_14, 0, x_1); -x_15 = 0; +lean_inc(x_3); +x_22 = lean_alloc_closure((void*)(l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__5___boxed), 13, 5); +lean_closure_set(x_22, 0, x_17); +lean_closure_set(x_22, 1, x_3); +lean_closure_set(x_22, 2, x_1); +lean_closure_set(x_22, 3, x_2); +lean_closure_set(x_22, 4, x_21); +x_23 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabBinders___rarg), 9, 2); +lean_closure_set(x_23, 0, x_20); +lean_closure_set(x_23, 1, x_22); +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_16 = l_Lean_Meta_forallTelescopeReducing___at_Lean_Meta_getParamNames___spec__2___rarg(x_13, x_14, x_15, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_16) == 0) +x_24 = l_Lean_Elab_Term_withAutoBoundImplicit___rarg(x_23, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_24) == 0) { -uint8_t x_17; -x_17 = !lean_is_exclusive(x_16); -if (x_17 == 0) +lean_object* x_25; lean_object* x_26; +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_ctor_set(x_5, 1, x_6); +lean_ctor_set(x_5, 0, x_25); { -lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; -x_18 = lean_ctor_get(x_16, 0); -x_19 = lean_ctor_get(x_16, 1); -x_20 = lean_unsigned_to_nat(0u); -x_21 = lean_nat_dec_eq(x_18, x_20); -lean_dec(x_18); -if (x_21 == 0) +lean_object* _tmp_4 = x_18; +lean_object* _tmp_5 = x_5; +lean_object* _tmp_12 = x_26; +x_5 = _tmp_4; +x_6 = _tmp_5; +x_13 = _tmp_12; +} +goto _start; +} +else { -lean_object* x_22; +uint8_t x_28; +lean_free_object(x_5); +lean_dec(x_18); lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_22 = l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__1___closed__2; -lean_ctor_set(x_16, 0, x_22); -return x_16; +x_28 = !lean_is_exclusive(x_24); +if (x_28 == 0) +{ +return x_24; } else { -lean_free_object(x_16); -lean_inc(x_2); -{ -lean_object* _tmp_2 = x_12; -lean_object* _tmp_3 = x_2; -lean_object* _tmp_8 = x_19; -x_3 = _tmp_2; -x_4 = _tmp_3; -x_9 = _tmp_8; +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; } -goto _start; } } else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; -x_24 = lean_ctor_get(x_16, 0); -x_25 = lean_ctor_get(x_16, 1); -lean_inc(x_25); -lean_inc(x_24); -lean_dec(x_16); -x_26 = lean_unsigned_to_nat(0u); -x_27 = lean_nat_dec_eq(x_24, x_26); -lean_dec(x_24); -if (x_27 == 0) -{ -lean_object* x_28; lean_object* x_29; -lean_dec(x_12); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); +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_5, 0); +x_33 = lean_ctor_get(x_5, 1); +lean_inc(x_33); +lean_inc(x_32); lean_dec(x_5); -lean_dec(x_2); -lean_dec(x_1); -x_28 = l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__1___closed__2; -x_29 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_29, 0, x_28); -lean_ctor_set(x_29, 1, x_25); -return x_29; -} -else -{ +x_34 = lean_ctor_get(x_32, 3); +lean_inc(x_34); +x_35 = l_Lean_Syntax_getArgs(x_34); +lean_dec(x_34); +x_36 = lean_box(x_4); lean_inc(x_2); +lean_inc(x_1); +lean_inc(x_3); +x_37 = lean_alloc_closure((void*)(l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__5___boxed), 13, 5); +lean_closure_set(x_37, 0, x_32); +lean_closure_set(x_37, 1, x_3); +lean_closure_set(x_37, 2, x_1); +lean_closure_set(x_37, 3, x_2); +lean_closure_set(x_37, 4, x_36); +x_38 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabBinders___rarg), 9, 2); +lean_closure_set(x_38, 0, x_35); +lean_closure_set(x_38, 1, x_37); +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_39 = l_Lean_Elab_Term_withAutoBoundImplicit___rarg(x_38, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_39) == 0) { -lean_object* _tmp_2 = x_12; -lean_object* _tmp_3 = x_2; -lean_object* _tmp_8 = x_25; -x_3 = _tmp_2; -x_4 = _tmp_3; -x_9 = _tmp_8; -} +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 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_42, 0, x_40); +lean_ctor_set(x_42, 1, x_6); +x_5 = x_33; +x_6 = x_42; +x_13 = x_41; goto _start; } -} -} else { -uint8_t x_31; +lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; +lean_dec(x_33); 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_31 = !lean_is_exclusive(x_16); -if (x_31 == 0) -{ -return x_16; +x_44 = lean_ctor_get(x_39, 0); +lean_inc(x_44); +x_45 = lean_ctor_get(x_39, 1); +lean_inc(x_45); +if (lean_is_exclusive(x_39)) { + lean_ctor_release(x_39, 0); + lean_ctor_release(x_39, 1); + x_46 = x_39; +} else { + lean_dec_ref(x_39); + x_46 = lean_box(0); } -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; +if (lean_is_scalar(x_46)) { + x_47 = lean_alloc_ctor(1, 2, 0); +} else { + x_47 = x_46; } +lean_ctor_set(x_47, 0, x_44); +lean_ctor_set(x_47, 1, x_45); +return x_47; } } } } -LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -if (lean_obj_tag(x_3) == 0) -{ -lean_object* x_10; -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_2); -lean_dec(x_1); -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_4); -lean_ctor_set(x_10, 1, x_9); -return x_10; } -else +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, 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_11; +lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_12 = lean_ctor_get(x_4, 0); +lean_inc(x_12); lean_dec(x_4); -x_11 = !lean_is_exclusive(x_3); -if (x_11 == 0) +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_array_get_size(x_3); +x_15 = !lean_is_exclusive(x_9); +if (x_15 == 0) { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_12 = lean_ctor_get(x_3, 0); -x_13 = lean_ctor_get(x_3, 1); -x_14 = lean_ctor_get(x_12, 2); -lean_inc(x_14); -lean_dec(x_12); +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_9, 5); +x_17 = l_Lean_replaceRef(x_13, x_16); +lean_dec(x_16); +lean_dec(x_13); +lean_ctor_set(x_9, 5, 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_n(x_2, 2); -lean_inc(x_1); -x_15 = l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__1(x_1, x_2, x_14, x_2, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_15) == 0) -{ -lean_object* x_16; lean_object* x_17; -x_16 = lean_ctor_get(x_15, 0); -lean_inc(x_16); -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -lean_dec(x_16); -if (lean_obj_tag(x_17) == 0) -{ -lean_object* x_18; -lean_free_object(x_3); -x_18 = lean_ctor_get(x_15, 1); -lean_inc(x_18); -lean_dec(x_15); lean_inc(x_2); +x_18 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isInductiveFamily(x_14, x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_18) == 0) { -lean_object* _tmp_2 = x_13; -lean_object* _tmp_3 = x_2; -lean_object* _tmp_8 = x_18; -x_3 = _tmp_2; -x_4 = _tmp_3; -x_9 = _tmp_8; -} -goto _start; +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; lean_object* x_25; +x_19 = lean_ctor_get(x_18, 0); +lean_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_12, 8); +lean_inc(x_21); +lean_dec(x_12); +x_22 = lean_array_to_list(x_21); +x_23 = lean_box(0); +x_24 = lean_unbox(x_19); +lean_dec(x_19); +x_25 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2(x_1, x_2, x_3, x_24, x_22, x_23, x_5, x_6, x_7, x_8, x_9, x_10, x_20); +return x_25; } else { -uint8_t x_20; -lean_dec(x_13); +uint8_t x_26; +lean_dec(x_9); +lean_dec(x_12); +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_2); lean_dec(x_1); -x_20 = !lean_is_exclusive(x_15); -if (x_20 == 0) -{ -lean_object* x_21; uint8_t x_22; -x_21 = lean_ctor_get(x_15, 0); -lean_dec(x_21); -x_22 = !lean_is_exclusive(x_17); -if (x_22 == 0) -{ -lean_object* x_23; -x_23 = lean_box(0); -lean_ctor_set_tag(x_3, 0); -lean_ctor_set(x_3, 1, x_23); -lean_ctor_set(x_3, 0, x_17); -lean_ctor_set(x_15, 0, x_3); -return x_15; -} -else +x_26 = !lean_is_exclusive(x_18); +if (x_26 == 0) { -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(1, 1, 0); -lean_ctor_set(x_25, 0, x_24); -x_26 = lean_box(0); -lean_ctor_set_tag(x_3, 0); -lean_ctor_set(x_3, 1, x_26); -lean_ctor_set(x_3, 0, x_25); -lean_ctor_set(x_15, 0, x_3); -return x_15; -} +return x_18; } 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_15, 1); -lean_inc(x_27); -lean_dec(x_15); -x_28 = lean_ctor_get(x_17, 0); +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_18, 0); +x_28 = lean_ctor_get(x_18, 1); lean_inc(x_28); -if (lean_is_exclusive(x_17)) { - lean_ctor_release(x_17, 0); - x_29 = x_17; -} else { - lean_dec_ref(x_17); - x_29 = lean_box(0); -} -if (lean_is_scalar(x_29)) { - x_30 = lean_alloc_ctor(1, 1, 0); -} else { - x_30 = x_29; -} -lean_ctor_set(x_30, 0, x_28); -x_31 = lean_box(0); -lean_ctor_set_tag(x_3, 0); -lean_ctor_set(x_3, 1, x_31); -lean_ctor_set(x_3, 0, x_30); -x_32 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_32, 0, x_3); -lean_ctor_set(x_32, 1, x_27); -return x_32; -} +lean_inc(x_27); +lean_dec(x_18); +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_27); +lean_ctor_set(x_29, 1, x_28); +return x_29; } } -else -{ -uint8_t x_33; -lean_free_object(x_3); -lean_dec(x_13); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_2); -lean_dec(x_1); -x_33 = !lean_is_exclusive(x_15); -if (x_33 == 0) -{ -return x_15; } else { -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_15, 0); -x_35 = lean_ctor_get(x_15, 1); -lean_inc(x_35); -lean_inc(x_34); -lean_dec(x_15); -x_36 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_36, 0, x_34); -lean_ctor_set(x_36, 1, x_35); -return x_36; -} -} -} -else -{ -lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_37 = lean_ctor_get(x_3, 0); -x_38 = lean_ctor_get(x_3, 1); +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; lean_object* x_42; uint8_t x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_30 = lean_ctor_get(x_9, 0); +x_31 = lean_ctor_get(x_9, 1); +x_32 = lean_ctor_get(x_9, 2); +x_33 = lean_ctor_get(x_9, 3); +x_34 = lean_ctor_get(x_9, 4); +x_35 = lean_ctor_get(x_9, 5); +x_36 = lean_ctor_get(x_9, 6); +x_37 = lean_ctor_get(x_9, 7); +x_38 = lean_ctor_get(x_9, 8); +x_39 = lean_ctor_get(x_9, 9); +x_40 = lean_ctor_get(x_9, 10); +x_41 = lean_ctor_get_uint8(x_9, sizeof(void*)*12); +x_42 = lean_ctor_get(x_9, 11); +x_43 = lean_ctor_get_uint8(x_9, sizeof(void*)*12 + 1); +lean_inc(x_42); +lean_inc(x_40); +lean_inc(x_39); lean_inc(x_38); lean_inc(x_37); -lean_dec(x_3); -x_39 = lean_ctor_get(x_37, 2); -lean_inc(x_39); -lean_dec(x_37); +lean_inc(x_36); +lean_inc(x_35); +lean_inc(x_34); +lean_inc(x_33); +lean_inc(x_32); +lean_inc(x_31); +lean_inc(x_30); +lean_dec(x_9); +x_44 = l_Lean_replaceRef(x_13, x_35); +lean_dec(x_35); +lean_dec(x_13); +x_45 = lean_alloc_ctor(0, 12, 2); +lean_ctor_set(x_45, 0, x_30); +lean_ctor_set(x_45, 1, x_31); +lean_ctor_set(x_45, 2, x_32); +lean_ctor_set(x_45, 3, x_33); +lean_ctor_set(x_45, 4, x_34); +lean_ctor_set(x_45, 5, x_44); +lean_ctor_set(x_45, 6, x_36); +lean_ctor_set(x_45, 7, x_37); +lean_ctor_set(x_45, 8, x_38); +lean_ctor_set(x_45, 9, x_39); +lean_ctor_set(x_45, 10, x_40); +lean_ctor_set(x_45, 11, x_42); +lean_ctor_set_uint8(x_45, sizeof(void*)*12, x_41); +lean_ctor_set_uint8(x_45, sizeof(void*)*12 + 1, x_43); +lean_inc(x_10); +lean_inc(x_45); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -lean_inc_n(x_2, 2); -lean_inc(x_1); -x_40 = l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__1(x_1, x_2, x_39, x_2, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_40) == 0) -{ -lean_object* x_41; lean_object* x_42; -x_41 = lean_ctor_get(x_40, 0); -lean_inc(x_41); -x_42 = lean_ctor_get(x_41, 0); -lean_inc(x_42); -lean_dec(x_41); -if (lean_obj_tag(x_42) == 0) -{ -lean_object* x_43; -x_43 = lean_ctor_get(x_40, 1); -lean_inc(x_43); -lean_dec(x_40); lean_inc(x_2); +x_46 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isInductiveFamily(x_14, x_2, x_5, x_6, x_7, x_8, x_45, x_10, x_11); +if (lean_obj_tag(x_46) == 0) { -lean_object* _tmp_2 = x_38; -lean_object* _tmp_3 = x_2; -lean_object* _tmp_8 = x_43; -x_3 = _tmp_2; -x_4 = _tmp_3; -x_9 = _tmp_8; -} -goto _start; +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; uint8_t x_52; lean_object* x_53; +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, 8); +lean_inc(x_49); +lean_dec(x_12); +x_50 = lean_array_to_list(x_49); +x_51 = lean_box(0); +x_52 = lean_unbox(x_47); +lean_dec(x_47); +x_53 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2(x_1, x_2, x_3, x_52, x_50, x_51, x_5, x_6, x_7, x_8, x_45, x_10, x_48); +return x_53; } else { -lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; -lean_dec(x_38); +lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; +lean_dec(x_45); +lean_dec(x_12); +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_2); lean_dec(x_1); -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; +x_54 = lean_ctor_get(x_46, 0); +lean_inc(x_54); +x_55 = lean_ctor_get(x_46, 1); +lean_inc(x_55); +if (lean_is_exclusive(x_46)) { + lean_ctor_release(x_46, 0); + lean_ctor_release(x_46, 1); + x_56 = x_46; } else { - lean_dec_ref(x_40); - x_46 = lean_box(0); + lean_dec_ref(x_46); + x_56 = lean_box(0); } -x_47 = lean_ctor_get(x_42, 0); -lean_inc(x_47); -if (lean_is_exclusive(x_42)) { - lean_ctor_release(x_42, 0); - x_48 = x_42; +if (lean_is_scalar(x_56)) { + x_57 = lean_alloc_ctor(1, 2, 0); } else { - lean_dec_ref(x_42); - x_48 = lean_box(0); + x_57 = x_56; } -if (lean_is_scalar(x_48)) { - x_49 = lean_alloc_ctor(1, 1, 0); -} else { - x_49 = x_48; +lean_ctor_set(x_57, 0, x_54); +lean_ctor_set(x_57, 1, x_55); +return x_57; } -lean_ctor_set(x_49, 0, x_47); -x_50 = lean_box(0); -x_51 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_51, 0, x_49); -lean_ctor_set(x_51, 1, x_50); -if (lean_is_scalar(x_46)) { - x_52 = lean_alloc_ctor(0, 2, 0); -} else { - x_52 = x_46; } -lean_ctor_set(x_52, 0, x_51); -lean_ctor_set(x_52, 1, x_45); -return x_52; } } -else +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: { -lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; -lean_dec(x_38); +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_Elab_Inductive_0__Lean_Elab_Command_elabCtors___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_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +uint8_t x_3; lean_object* x_4; +x_3 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___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_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_2); +lean_dec(x_4); +lean_dec(x_3); lean_dec(x_1); -x_53 = lean_ctor_get(x_40, 0); -lean_inc(x_53); -x_54 = lean_ctor_get(x_40, 1); -lean_inc(x_54); -if (lean_is_exclusive(x_40)) { - lean_ctor_release(x_40, 0); - lean_ctor_release(x_40, 1); - x_55 = x_40; -} else { - lean_dec_ref(x_40); - x_55 = lean_box(0); +return x_11; } -if (lean_is_scalar(x_55)) { - x_56 = lean_alloc_ctor(1, 2, 0); -} else { - x_56 = x_55; } -lean_ctor_set(x_56, 0, x_53); -lean_ctor_set(x_56, 1, x_54); -return x_56; +LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; +x_15 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_2); +return x_15; +} } +LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___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_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +x_12 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_1); +return x_12; } } +LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___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) { +_start: +{ +uint8_t x_14; lean_object* x_15; +x_14 = lean_unbox(x_5); +lean_dec(x_5); +x_15 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___lambda__5(x_1, x_2, x_3, x_4, x_14, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +return x_15; } } -LEAN_EXPORT lean_object* l_List_foldl___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__3(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -if (lean_obj_tag(x_2) == 0) +uint8_t x_14; lean_object* x_15; +x_14 = lean_unbox(x_4); +lean_dec(x_4); +x_15 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___spec__2(x_1, x_2, x_3, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +return x_15; +} +} +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___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: { -return x_1; +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_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_is_exclusive(x_12); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_14 = lean_ctor_get(x_12, 0); +x_15 = lean_ctor_get(x_12, 1); +x_16 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(x_14, x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_15); +lean_dec(x_2); +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_12, 1, x_18); +lean_ctor_set(x_12, 0, x_11); +lean_ctor_set_tag(x_16, 1); +lean_ctor_set(x_16, 0, x_12); +return x_16; } else { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; -x_3 = lean_ctor_get(x_2, 0); -x_4 = lean_ctor_get(x_2, 1); -x_5 = lean_ctor_get(x_3, 2); -x_6 = lean_unsigned_to_nat(0u); -x_7 = l_List_lengthTRAux___rarg(x_5, x_6); -x_8 = lean_nat_dec_le(x_1, x_7); -if (x_8 == 0) -{ -lean_dec(x_7); -x_2 = x_4; -goto _start; +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_12, 1, x_19); +lean_ctor_set(x_12, 0, x_11); +x_21 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_21, 0, x_12); +lean_ctor_set(x_21, 1, x_20); +return x_21; +} } else { -lean_dec(x_1); -x_1 = x_7; -x_2 = x_4; -goto _start; +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +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 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(x_22, x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_23); +lean_dec(x_2); +x_25 = lean_ctor_get(x_24, 0); +lean_inc(x_25); +x_26 = lean_ctor_get(x_24, 1); +lean_inc(x_26); +if (lean_is_exclusive(x_24)) { + lean_ctor_release(x_24, 0); + lean_ctor_release(x_24, 1); + x_27 = x_24; +} else { + lean_dec_ref(x_24); + x_27 = lean_box(0); +} +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_11); +lean_ctor_set(x_28, 1, x_25); +if (lean_is_scalar(x_27)) { + x_29 = lean_alloc_ctor(1, 2, 0); +} else { + x_29 = x_27; + lean_ctor_set_tag(x_29, 1); } +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_26); +return x_29; } } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___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) { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___lambda__1___closed__1() { _start: { -uint8_t x_7; lean_object* x_8; lean_object* x_9; -x_7 = 0; -x_8 = lean_box(x_7); -x_9 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_9, 0, x_8); -lean_ctor_set(x_9, 1, x_6); -return x_9; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("unexpected inductive type resulting type", 40, 40); +return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___lambda__2___closed__1() { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___lambda__1___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___lambda__1___boxed), 6, 0); -return x_1; +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___lambda__1___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___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_object* x_10; -x_9 = l_Lean_Elab_Command_withCtorRef___rarg___closed__1; +lean_object* x_10; +lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -lean_inc(x_4); -x_10 = l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__2(x_1, x_9, x_2, x_9, x_4, x_5, x_6, x_7, x_8); +x_10 = l_Lean_Meta_whnfD(x_2, 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_11; x_11 = lean_ctor_get(x_10, 0); lean_inc(x_11); -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); -lean_dec(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; -x_13 = lean_ctor_get(x_10, 1); -lean_inc(x_13); -lean_dec(x_10); -x_14 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___lambda__2___closed__1; -x_15 = lean_box(0); -x_16 = lean_apply_6(x_14, x_15, x_4, x_5, x_6, x_7, x_13); -return x_16; -} -else +if (lean_obj_tag(x_11) == 3) { -uint8_t x_17; +uint8_t x_12; +lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); -x_17 = !lean_is_exclusive(x_10); -if (x_17 == 0) +lean_dec(x_3); +x_12 = !lean_is_exclusive(x_10); +if (x_12 == 0) { -lean_object* x_18; lean_object* x_19; -x_18 = lean_ctor_get(x_10, 0); -lean_dec(x_18); -x_19 = lean_ctor_get(x_12, 0); -lean_inc(x_19); -lean_dec(x_12); -lean_ctor_set(x_10, 0, x_19); +lean_object* x_13; lean_object* x_14; +x_13 = lean_ctor_get(x_10, 0); +lean_dec(x_13); +x_14 = lean_ctor_get(x_11, 0); +lean_inc(x_14); +lean_dec(x_11); +lean_ctor_set(x_10, 0, x_14); return x_10; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_10, 1); -lean_inc(x_20); +lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_15 = lean_ctor_get(x_10, 1); +lean_inc(x_15); lean_dec(x_10); -x_21 = lean_ctor_get(x_12, 0); -lean_inc(x_21); -lean_dec(x_12); -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_21); -lean_ctor_set(x_22, 1, x_20); -return x_22; +x_16 = lean_ctor_get(x_11, 0); +lean_inc(x_16); +lean_dec(x_11); +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_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_18 = lean_ctor_get(x_10, 1); +lean_inc(x_18); +lean_dec(x_10); +x_19 = l_Lean_indentExpr(x_11); +x_20 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___lambda__1___closed__2; +x_21 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_21, 0, x_20); +lean_ctor_set(x_21, 1, x_19); +x_22 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +x_23 = lean_alloc_ctor(7, 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_Inductive_0__Lean_Elab_Command_getResultingUniverse___spec__1(x_23, x_3, x_4, x_5, x_6, x_7, x_8, x_18); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +return x_24; +} } else { -uint8_t x_23; +uint8_t x_25; +lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); -x_23 = !lean_is_exclusive(x_10); -if (x_23 == 0) +lean_dec(x_3); +x_25 = !lean_is_exclusive(x_10); +if (x_25 == 0) { return x_10; } else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_10, 0); -x_25 = lean_ctor_get(x_10, 1); -lean_inc(x_25); -lean_inc(x_24); +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_10, 0); +x_27 = lean_ctor_get(x_10, 1); +lean_inc(x_27); +lean_inc(x_26); lean_dec(x_10); -x_26 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_26, 0, x_24); -lean_ctor_set(x_26, 1, x_25); -return x_26; +x_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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate(lean_object* x_1, 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_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___closed__1() { _start: { -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_List_foldl___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__3(x_8, x_2); -x_10 = lean_unsigned_to_nat(1u); -x_11 = lean_nat_dec_eq(x_9, 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_6); -lean_dec(x_5); -lean_dec(x_4); -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_7); -return x_14; -} -else -{ -lean_object* x_15; lean_object* x_16; -x_15 = lean_box(0); -x_16 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___lambda__2(x_1, x_2, x_15, x_3, x_4, x_5, x_6, x_7); -return x_16; -} +lean_object* x_1; +x_1 = lean_mk_string_unchecked("unexpected empty inductive declaration", 38, 38); +return x_1; } } -LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___closed__2() { _start: { -lean_object* x_9; -x_9 = l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_9; +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l_List_foldl___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__3___boxed(lean_object* x_1, lean_object* x_2) { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___closed__3() { _start: { -lean_object* x_3; -x_3 = l_List_foldl___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__3(x_1, x_2); -lean_dec(x_2); -return x_3; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___lambda__1___boxed), 9, 0); +return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___lambda__1___boxed(lean_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_Inductive_0__Lean_Elab_Command_getResultingUniverse(lean_object* x_1, lean_object* x_2, lean_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_Inductive_0__Lean_Elab_Command_isPropCandidate___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6); +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_9; lean_object* x_10; +x_9 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___closed__2; +x_10 = l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___spec__1(x_9, 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_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; lean_object* x_15; +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); lean_dec(x_1); -return x_7; +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___closed__3; +x_14 = 0; +x_15 = l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___spec__1___rarg(x_12, x_13, x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +return x_15; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +} +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___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); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_assignLevelMVar___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; -x_10 = lean_st_ref_take(x_6, x_9); -x_11 = lean_ctor_get(x_10, 0); +lean_object* x_10; +x_10 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___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_1); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_shouldInferResultUniverse___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; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; +x_9 = lean_st_ref_get(x_5, 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); -x_12 = lean_ctor_get(x_11, 0); +lean_dec(x_9); +x_12 = lean_ctor_get(x_10, 0); lean_inc(x_12); -x_13 = lean_ctor_get(x_10, 1); -lean_inc(x_13); lean_dec(x_10); -x_14 = !lean_is_exclusive(x_11); -if (x_14 == 0) -{ -lean_object* x_15; uint8_t x_16; -x_15 = lean_ctor_get(x_11, 0); -lean_dec(x_15); -x_16 = !lean_is_exclusive(x_12); -if (x_16 == 0) +x_13 = lean_instantiate_level_mvars(x_12, x_1); +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_13, 1); +lean_inc(x_15); +lean_dec(x_13); +x_16 = lean_st_ref_take(x_5, x_11); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +x_19 = !lean_is_exclusive(x_17); +if (x_19 == 0) { -lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; -x_17 = lean_ctor_get(x_12, 6); -x_18 = l_Lean_PersistentHashMap_insert___at_Lean_assignLevelMVar___spec__1(x_17, x_1, x_2); -lean_ctor_set(x_12, 6, x_18); -x_19 = lean_st_ref_set(x_6, x_11, x_13); -x_20 = !lean_is_exclusive(x_19); -if (x_20 == 0) +lean_object* x_20; lean_object* x_21; uint8_t x_22; +x_20 = lean_ctor_get(x_17, 0); +lean_dec(x_20); +lean_ctor_set(x_17, 0, x_14); +x_21 = lean_st_ref_set(x_5, x_17, x_18); +x_22 = !lean_is_exclusive(x_21); +if (x_22 == 0) { -lean_object* x_21; lean_object* x_22; -x_21 = lean_ctor_get(x_19, 0); -lean_dec(x_21); -x_22 = lean_box(0); -lean_ctor_set(x_19, 0, x_22); -return x_19; +lean_object* x_23; +x_23 = lean_ctor_get(x_21, 0); +lean_dec(x_23); +lean_ctor_set(x_21, 0, x_15); +return x_21; } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_19, 1); -lean_inc(x_23); -lean_dec(x_19); -x_24 = lean_box(0); +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_21, 1); +lean_inc(x_24); +lean_dec(x_21); 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, 0, x_15); +lean_ctor_set(x_25, 1, x_24); 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_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_26 = lean_ctor_get(x_12, 0); -x_27 = lean_ctor_get(x_12, 1); -x_28 = lean_ctor_get(x_12, 2); -x_29 = lean_ctor_get(x_12, 3); -x_30 = lean_ctor_get(x_12, 4); -x_31 = lean_ctor_get(x_12, 5); -x_32 = lean_ctor_get(x_12, 6); -x_33 = lean_ctor_get(x_12, 7); -x_34 = lean_ctor_get(x_12, 8); -lean_inc(x_34); -lean_inc(x_33); -lean_inc(x_32); -lean_inc(x_31); -lean_inc(x_30); +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_26 = lean_ctor_get(x_17, 1); +x_27 = lean_ctor_get(x_17, 2); +x_28 = lean_ctor_get(x_17, 3); +x_29 = lean_ctor_get(x_17, 4); lean_inc(x_29); lean_inc(x_28); lean_inc(x_27); lean_inc(x_26); -lean_dec(x_12); -x_35 = l_Lean_PersistentHashMap_insert___at_Lean_assignLevelMVar___spec__1(x_32, x_1, x_2); -x_36 = lean_alloc_ctor(0, 9, 0); -lean_ctor_set(x_36, 0, x_26); -lean_ctor_set(x_36, 1, x_27); -lean_ctor_set(x_36, 2, x_28); -lean_ctor_set(x_36, 3, x_29); -lean_ctor_set(x_36, 4, x_30); -lean_ctor_set(x_36, 5, x_31); -lean_ctor_set(x_36, 6, x_35); -lean_ctor_set(x_36, 7, x_33); -lean_ctor_set(x_36, 8, x_34); -lean_ctor_set(x_11, 0, x_36); -x_37 = lean_st_ref_set(x_6, x_11, x_13); -x_38 = lean_ctor_get(x_37, 1); -lean_inc(x_38); -if (lean_is_exclusive(x_37)) { - lean_ctor_release(x_37, 0); - lean_ctor_release(x_37, 1); - x_39 = x_37; -} else { - lean_dec_ref(x_37); - x_39 = lean_box(0); -} -x_40 = lean_box(0); -if (lean_is_scalar(x_39)) { - x_41 = lean_alloc_ctor(0, 2, 0); -} else { - x_41 = x_39; -} -lean_ctor_set(x_41, 0, x_40); -lean_ctor_set(x_41, 1, x_38); -return x_41; -} -} -else -{ -lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; -x_42 = lean_ctor_get(x_11, 1); -x_43 = lean_ctor_get(x_11, 2); -x_44 = lean_ctor_get(x_11, 3); -x_45 = lean_ctor_get(x_11, 4); -lean_inc(x_45); -lean_inc(x_44); -lean_inc(x_43); -lean_inc(x_42); -lean_dec(x_11); -x_46 = lean_ctor_get(x_12, 0); -lean_inc(x_46); -x_47 = lean_ctor_get(x_12, 1); -lean_inc(x_47); -x_48 = lean_ctor_get(x_12, 2); -lean_inc(x_48); -x_49 = lean_ctor_get(x_12, 3); -lean_inc(x_49); -x_50 = lean_ctor_get(x_12, 4); -lean_inc(x_50); -x_51 = lean_ctor_get(x_12, 5); -lean_inc(x_51); -x_52 = lean_ctor_get(x_12, 6); -lean_inc(x_52); -x_53 = lean_ctor_get(x_12, 7); -lean_inc(x_53); -x_54 = lean_ctor_get(x_12, 8); -lean_inc(x_54); -if (lean_is_exclusive(x_12)) { - lean_ctor_release(x_12, 0); - lean_ctor_release(x_12, 1); - lean_ctor_release(x_12, 2); - lean_ctor_release(x_12, 3); - lean_ctor_release(x_12, 4); - lean_ctor_release(x_12, 5); - lean_ctor_release(x_12, 6); - lean_ctor_release(x_12, 7); - lean_ctor_release(x_12, 8); - x_55 = x_12; -} else { - lean_dec_ref(x_12); - x_55 = lean_box(0); -} -x_56 = l_Lean_PersistentHashMap_insert___at_Lean_assignLevelMVar___spec__1(x_52, x_1, x_2); -if (lean_is_scalar(x_55)) { - x_57 = lean_alloc_ctor(0, 9, 0); -} else { - x_57 = x_55; -} -lean_ctor_set(x_57, 0, x_46); -lean_ctor_set(x_57, 1, x_47); -lean_ctor_set(x_57, 2, x_48); -lean_ctor_set(x_57, 3, x_49); -lean_ctor_set(x_57, 4, x_50); -lean_ctor_set(x_57, 5, x_51); -lean_ctor_set(x_57, 6, x_56); -lean_ctor_set(x_57, 7, x_53); -lean_ctor_set(x_57, 8, x_54); -x_58 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_58, 0, x_57); -lean_ctor_set(x_58, 1, x_42); -lean_ctor_set(x_58, 2, x_43); -lean_ctor_set(x_58, 3, x_44); -lean_ctor_set(x_58, 4, x_45); -x_59 = lean_st_ref_set(x_6, x_58, x_13); -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; +lean_dec(x_17); +x_30 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_30, 0, x_14); +lean_ctor_set(x_30, 1, x_26); +lean_ctor_set(x_30, 2, x_27); +lean_ctor_set(x_30, 3, x_28); +lean_ctor_set(x_30, 4, x_29); +x_31 = lean_st_ref_set(x_5, x_30, x_18); +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; } else { - lean_dec_ref(x_59); - x_61 = lean_box(0); + lean_dec_ref(x_31); + x_33 = lean_box(0); } -x_62 = lean_box(0); -if (lean_is_scalar(x_61)) { - x_63 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_33)) { + x_34 = lean_alloc_ctor(0, 2, 0); } else { - x_63 = x_61; + x_34 = x_33; } -lean_ctor_set(x_63, 0, x_62); -lean_ctor_set(x_63, 1, x_60); -return x_63; +lean_ctor_set(x_34, 0, x_15); +lean_ctor_set(x_34, 1, x_32); +return x_34; } } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_shouldInferResultUniverse___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -if (lean_obj_tag(x_1) == 0) +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_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_is_exclusive(x_12); +if (x_13 == 0) { -lean_object* x_10; lean_object* x_11; -x_10 = l_List_reverse___rarg(x_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); -return x_11; +lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_14 = lean_ctor_get(x_12, 0); +x_15 = lean_ctor_get(x_12, 1); +x_16 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(x_14, x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_15); +lean_dec(x_2); +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_12, 1, x_18); +lean_ctor_set(x_12, 0, x_11); +lean_ctor_set_tag(x_16, 1); +lean_ctor_set(x_16, 0, x_12); +return x_16; } else { -uint8_t x_12; -x_12 = !lean_is_exclusive(x_1); -if (x_12 == 0) -{ -lean_object* x_13; uint8_t x_14; -x_13 = lean_ctor_get(x_1, 0); -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_1, 1); -x_16 = lean_ctor_get(x_13, 1); -x_17 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_16, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -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_16, 0); +x_20 = lean_ctor_get(x_16, 1); +lean_inc(x_20); lean_inc(x_19); -lean_dec(x_17); -lean_ctor_set(x_13, 1, x_18); -lean_ctor_set(x_1, 1, x_2); -{ -lean_object* _tmp_0 = x_15; -lean_object* _tmp_1 = x_1; -lean_object* _tmp_8 = x_19; -x_1 = _tmp_0; -x_2 = _tmp_1; -x_9 = _tmp_8; +lean_dec(x_16); +lean_ctor_set(x_12, 1, x_19); +lean_ctor_set(x_12, 0, x_11); +x_21 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_21, 0, x_12); +lean_ctor_set(x_21, 1, x_20); +return x_21; } -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; -x_21 = lean_ctor_get(x_1, 1); -x_22 = lean_ctor_get(x_13, 0); -x_23 = lean_ctor_get(x_13, 1); +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_22 = lean_ctor_get(x_12, 0); +x_23 = lean_ctor_get(x_12, 1); lean_inc(x_23); lean_inc(x_22); -lean_dec(x_13); -x_24 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_23, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_12); +x_24 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(x_22, x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_23); +lean_dec(x_2); x_25 = lean_ctor_get(x_24, 0); lean_inc(x_25); x_26 = lean_ctor_get(x_24, 1); lean_inc(x_26); -lean_dec(x_24); -x_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_22); -lean_ctor_set(x_27, 1, x_25); -lean_ctor_set(x_1, 1, x_2); -lean_ctor_set(x_1, 0, x_27); -{ -lean_object* _tmp_0 = x_21; -lean_object* _tmp_1 = x_1; -lean_object* _tmp_8 = x_26; -x_1 = _tmp_0; -x_2 = _tmp_1; -x_9 = _tmp_8; +if (lean_is_exclusive(x_24)) { + lean_ctor_release(x_24, 0); + lean_ctor_release(x_24, 1); + x_27 = x_24; +} else { + lean_dec_ref(x_24); + x_27 = lean_box(0); } -goto _start; +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_11); +lean_ctor_set(x_28, 1, x_25); +if (lean_is_scalar(x_27)) { + x_29 = lean_alloc_ctor(1, 2, 0); +} else { + x_29 = x_27; + lean_ctor_set_tag(x_29, 1); } +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_26); +return x_29; } -else -{ -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_29 = lean_ctor_get(x_1, 0); -x_30 = lean_ctor_get(x_1, 1); -lean_inc(x_30); -lean_inc(x_29); -lean_dec(x_1); -x_31 = lean_ctor_get(x_29, 0); -lean_inc(x_31); -x_32 = lean_ctor_get(x_29, 1); -lean_inc(x_32); -if (lean_is_exclusive(x_29)) { - lean_ctor_release(x_29, 0); - lean_ctor_release(x_29, 1); - x_33 = x_29; -} else { - lean_dec_ref(x_29); - x_33 = lean_box(0); } -x_34 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_32, 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); -if (lean_is_scalar(x_33)) { - x_37 = lean_alloc_ctor(0, 2, 0); -} else { - x_37 = x_33; } -lean_ctor_set(x_37, 0, x_31); -lean_ctor_set(x_37, 1, x_35); -x_38 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_38, 0, x_37); -lean_ctor_set(x_38, 1, x_2); -x_1 = x_30; -x_2 = x_38; -x_9 = x_36; -goto _start; +static lean_object* _init_l_Lean_Elab_Command_shouldInferResultUniverse___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("cannot infer resulting universe level of inductive datatype, given level contains metavariables ", 96, 96); +return x_1; } } +static lean_object* _init_l_Lean_Elab_Command_shouldInferResultUniverse___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_shouldInferResultUniverse___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___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) { +static lean_object* _init_l_Lean_Elab_Command_shouldInferResultUniverse___closed__3() { _start: { -if (lean_obj_tag(x_1) == 0) +lean_object* x_1; +x_1 = lean_mk_string_unchecked(", provide universe explicitly", 29, 29); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Command_shouldInferResultUniverse___closed__4() { +_start: { -lean_object* x_10; lean_object* x_11; -x_10 = l_List_reverse___rarg(x_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); -return x_11; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_shouldInferResultUniverse___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } -else +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_shouldInferResultUniverse(lean_object* x_1, lean_object* x_2, lean_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_12; -x_12 = !lean_is_exclusive(x_1); -if (x_12 == 0) +lean_object* x_9; uint8_t x_10; +x_9 = l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_shouldInferResultUniverse___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_10 = !lean_is_exclusive(x_9); +if (x_10 == 0) { -lean_object* x_13; uint8_t x_14; -x_13 = lean_ctor_get(x_1, 0); -x_14 = !lean_is_exclusive(x_13); -if (x_14 == 0) +lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_11 = lean_ctor_get(x_9, 0); +x_12 = lean_ctor_get(x_9, 1); +x_13 = l_Lean_Level_hasMVar(x_11); +if (x_13 == 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_1, 1); -x_16 = lean_ctor_get(x_13, 1); -x_17 = lean_ctor_get(x_13, 2); -x_18 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_16, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -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_box(0); -x_22 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___spec__2(x_17, x_21, x_3, x_4, x_5, x_6, x_7, x_8, 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_ctor_set(x_13, 2, x_23); -lean_ctor_set(x_13, 1, x_19); -lean_ctor_set(x_1, 1, x_2); +lean_object* x_14; +lean_dec(x_11); +lean_dec(x_2); +x_14 = lean_box(0); +lean_ctor_set(x_9, 0, x_14); +return x_9; +} +else { -lean_object* _tmp_0 = x_15; -lean_object* _tmp_1 = x_1; -lean_object* _tmp_8 = x_24; -x_1 = _tmp_0; -x_2 = _tmp_1; -x_9 = _tmp_8; +lean_object* x_15; +x_15 = l_Lean_Level_getLevelOffset(x_11); +if (lean_obj_tag(x_15) == 5) +{ +lean_object* x_16; lean_object* x_17; +lean_dec(x_11); +lean_dec(x_2); +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +lean_dec(x_15); +x_17 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_17, 0, x_16); +lean_ctor_set(x_9, 0, x_17); +return x_9; +} +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_dec(x_15); +lean_free_object(x_9); +x_18 = l_Lean_Expr_sort___override(x_11); +x_19 = l_Lean_MessageData_ofExpr(x_18); +x_20 = l_Lean_Elab_Command_shouldInferResultUniverse___closed__2; +x_21 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_21, 0, x_20); +lean_ctor_set(x_21, 1, x_19); +x_22 = l_Lean_Elab_Command_shouldInferResultUniverse___closed__4; +x_23 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_23, 0, x_21); +lean_ctor_set(x_23, 1, x_22); +x_24 = l_Lean_throwError___at_Lean_Elab_Command_shouldInferResultUniverse___spec__2(x_23, x_2, x_3, x_4, x_5, x_6, x_7, x_12); +return x_24; +} } -goto _start; } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_26 = lean_ctor_get(x_1, 1); -x_27 = lean_ctor_get(x_13, 0); -x_28 = lean_ctor_get(x_13, 1); -x_29 = lean_ctor_get(x_13, 2); -lean_inc(x_29); -lean_inc(x_28); -lean_inc(x_27); -lean_dec(x_13); -x_30 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_28, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_object* x_25; lean_object* x_26; uint8_t x_27; +x_25 = lean_ctor_get(x_9, 0); +x_26 = lean_ctor_get(x_9, 1); +lean_inc(x_26); +lean_inc(x_25); +lean_dec(x_9); +x_27 = l_Lean_Level_hasMVar(x_25); +if (x_27 == 0) +{ +lean_object* x_28; lean_object* x_29; +lean_dec(x_25); +lean_dec(x_2); +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_26); +return x_29; +} +else +{ +lean_object* x_30; +x_30 = l_Lean_Level_getLevelOffset(x_25); +if (lean_obj_tag(x_30) == 5) +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; +lean_dec(x_25); +lean_dec(x_2); 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_box(0); -x_34 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___spec__2(x_29, x_33, x_3, x_4, x_5, x_6, x_7, x_8, 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_alloc_ctor(0, 3, 0); -lean_ctor_set(x_37, 0, x_27); -lean_ctor_set(x_37, 1, x_31); -lean_ctor_set(x_37, 2, x_35); -lean_ctor_set(x_1, 1, x_2); -lean_ctor_set(x_1, 0, x_37); +x_32 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_32, 0, x_31); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_26); +return x_33; +} +else { -lean_object* _tmp_0 = x_26; -lean_object* _tmp_1 = x_1; -lean_object* _tmp_8 = x_36; -x_1 = _tmp_0; -x_2 = _tmp_1; -x_9 = _tmp_8; +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_dec(x_30); +x_34 = l_Lean_Expr_sort___override(x_25); +x_35 = l_Lean_MessageData_ofExpr(x_34); +x_36 = l_Lean_Elab_Command_shouldInferResultUniverse___closed__2; +x_37 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_37, 0, x_36); +lean_ctor_set(x_37, 1, x_35); +x_38 = l_Lean_Elab_Command_shouldInferResultUniverse___closed__4; +x_39 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_39, 0, x_37); +lean_ctor_set(x_39, 1, x_38); +x_40 = l_Lean_throwError___at_Lean_Elab_Command_shouldInferResultUniverse___spec__2(x_39, x_2, x_3, x_4, x_5, x_6, x_7, x_26); +return x_40; } -goto _start; } } -else +} +} +LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_shouldInferResultUniverse___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_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_39 = lean_ctor_get(x_1, 0); -x_40 = lean_ctor_get(x_1, 1); -lean_inc(x_40); -lean_inc(x_39); -lean_dec(x_1); -x_41 = lean_ctor_get(x_39, 0); -lean_inc(x_41); -x_42 = lean_ctor_get(x_39, 1); -lean_inc(x_42); -x_43 = lean_ctor_get(x_39, 2); -lean_inc(x_43); -if (lean_is_exclusive(x_39)) { - lean_ctor_release(x_39, 0); - lean_ctor_release(x_39, 1); - lean_ctor_release(x_39, 2); - x_44 = x_39; -} else { - lean_dec_ref(x_39); - x_44 = lean_box(0); +lean_object* x_9; +x_9 = l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_shouldInferResultUniverse___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; } -x_45 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_42, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -x_46 = lean_ctor_get(x_45, 0); -lean_inc(x_46); -x_47 = lean_ctor_get(x_45, 1); -lean_inc(x_47); -lean_dec(x_45); -x_48 = lean_box(0); -x_49 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___spec__2(x_43, x_48, x_3, x_4, x_5, x_6, x_7, x_8, x_47); -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); -if (lean_is_scalar(x_44)) { - x_52 = lean_alloc_ctor(0, 3, 0); -} else { - x_52 = x_44; } -lean_ctor_set(x_52, 0, x_41); -lean_ctor_set(x_52, 1, x_46); -lean_ctor_set(x_52, 2, x_50); -x_53 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_53, 0, x_52); -lean_ctor_set(x_53, 1, x_2); -x_1 = x_40; -x_2 = x_53; -x_9 = x_51; -goto _start; +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_shouldInferResultUniverse___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) { +_start: +{ +lean_object* x_9; +x_9 = l_Lean_throwError___at_Lean_Elab_Command_shouldInferResultUniverse___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_9; } } +LEAN_EXPORT lean_object* l_Lean_Elab_Command_shouldInferResultUniverse___boxed(lean_object* x_1, lean_object* x_2, lean_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_Command_shouldInferResultUniverse(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_9; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___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 uint8_t l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27___spec__1(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_14; -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_2); -x_14 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate(x_1, x_2, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_14) == 0) +if (lean_obj_tag(x_1) == 0) { -lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -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_Lean_Elab_Command_mkResultUniverse(x_3, x_4, x_17); -x_19 = l_Lean_Level_mvarId_x21(x_5); -x_20 = l_Lean_assignLevelMVar___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___spec__1(x_19, x_18, x_7, x_8, x_9, x_10, x_11, x_12, x_16); -x_21 = lean_ctor_get(x_20, 1); -lean_inc(x_21); -lean_dec(x_20); -x_22 = lean_box(0); -x_23 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___spec__3(x_2, x_22, x_7, x_8, x_9, x_10, x_11, x_12, x_21); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -return x_23; +if (lean_obj_tag(x_2) == 0) +{ +uint8_t x_3; +x_3 = 1; +return x_3; } else { -uint8_t x_24; -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_3); -lean_dec(x_2); -x_24 = !lean_is_exclusive(x_14); -if (x_24 == 0) +uint8_t x_4; +x_4 = 0; +return x_4; +} +} +else { -return x_14; +if (lean_obj_tag(x_2) == 0) +{ +uint8_t x_5; +x_5 = 0; +return x_5; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_14, 0); -x_26 = lean_ctor_get(x_14, 1); -lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_14); -x_27 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_26); -return x_27; +lean_object* x_6; lean_object* x_7; uint8_t x_8; +x_6 = lean_ctor_get(x_1, 0); +x_7 = lean_ctor_get(x_2, 0); +x_8 = lean_name_eq(x_6, x_7); +return x_8; } } } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__1() { +LEAN_EXPORT uint8_t l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27___lambda__1(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("updateResultingUniverse us: ", 28, 28); -return x_1; +lean_object* x_3; uint8_t x_4; +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +x_4 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27___spec__1(x_1, x_3); +lean_dec(x_3); +return x_4; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__2() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_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) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +lean_object* x_10; lean_object* x_11; +x_10 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27___lambda__1___boxed), 2, 1); +lean_closure_set(x_10, 0, x_1); +x_11 = l_Lean_Elab_Term_levelMVarToParam(x_2, x_10, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_11; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__3() { +LEAN_EXPORT lean_object* l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27___spec__1___boxed(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked(", r: ", 5, 5); -return x_1; +uint8_t x_3; lean_object* x_4; +x_3 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27___spec__1(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +x_4 = lean_box(x_3); +return x_4; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__4() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__3; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +uint8_t x_3; lean_object* x_4; +x_3 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27___lambda__1(x_1, x_2); +lean_dec(x_1); +x_4 = lean_box(x_3); +return x_4; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__5() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_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) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked(", rOffset: ", 11, 11); -return x_1; +lean_object* x_10; +x_10 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_10; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__6() { +LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam___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_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__5; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_11; lean_object* x_12; +lean_dec(x_1); +x_11 = l_List_reverse___rarg(x_3); +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_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___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: +else { -lean_object* x_14; -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_2); -x_14 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses(x_1, x_2, x_3, x_4, x_5, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_14) == 0) +uint8_t x_13; +x_13 = !lean_is_exclusive(x_2); +if (x_13 == 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; -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_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__3; -x_18 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_17, x_7, x_8, x_9, x_10, x_11, x_12, x_16); +lean_object* x_14; uint8_t x_15; +x_14 = lean_ctor_get(x_2, 0); +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; +x_16 = lean_ctor_get(x_2, 1); +x_17 = lean_ctor_get(x_14, 1); +lean_inc(x_1); +x_18 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27(x_1, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10); x_19 = lean_ctor_get(x_18, 0); lean_inc(x_19); -x_20 = lean_unbox(x_19); -lean_dec(x_19); -if (x_20 == 0) -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_18, 1); -lean_inc(x_21); +x_20 = lean_ctor_get(x_18, 1); +lean_inc(x_20); lean_dec(x_18); -x_22 = lean_box(0); -x_23 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__1(x_4, x_5, x_15, x_3, x_2, x_22, x_7, x_8, x_9, x_10, x_11, x_12, x_21); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_2); -lean_dec(x_3); -return x_23; -} -else -{ -uint8_t x_24; -x_24 = !lean_is_exclusive(x_18); -if (x_24 == 0) +lean_ctor_set(x_14, 1, x_19); +lean_ctor_set(x_2, 1, x_3); { -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_25 = lean_ctor_get(x_18, 1); -x_26 = lean_ctor_get(x_18, 0); -lean_dec(x_26); -lean_inc(x_15); -x_27 = lean_array_to_list(x_15); -x_28 = lean_box(0); -x_29 = l_List_mapTR_loop___at_Lean_Meta_Match_mkMatcher___spec__6(x_27, x_28); -x_30 = l_Lean_MessageData_ofList(x_29); -x_31 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__2; -lean_ctor_set_tag(x_18, 7); -lean_ctor_set(x_18, 1, x_30); -lean_ctor_set(x_18, 0, x_31); -x_32 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__4; -x_33 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_33, 0, x_18); -lean_ctor_set(x_33, 1, x_32); -lean_inc(x_2); -x_34 = l_Lean_MessageData_ofLevel(x_2); -x_35 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_35, 0, x_33); -lean_ctor_set(x_35, 1, x_34); -x_36 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__6; -x_37 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -lean_inc(x_3); -x_38 = l___private_Init_Data_Repr_0__Nat_reprFast(x_3); -x_39 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_39, 0, x_38); -x_40 = l_Lean_MessageData_ofFormat(x_39); -x_41 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_41, 0, x_37); -lean_ctor_set(x_41, 1, x_40); -x_42 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5; -x_43 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_43, 0, x_41); -lean_ctor_set(x_43, 1, x_42); -x_44 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_17, x_43, x_7, x_8, x_9, x_10, x_11, x_12, x_25); -x_45 = lean_ctor_get(x_44, 0); -lean_inc(x_45); -x_46 = lean_ctor_get(x_44, 1); -lean_inc(x_46); -lean_dec(x_44); -x_47 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__1(x_4, x_5, x_15, x_3, x_2, x_45, x_7, x_8, x_9, x_10, x_11, x_12, x_46); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_45); -lean_dec(x_2); -lean_dec(x_3); -return x_47; +lean_object* _tmp_1 = x_16; +lean_object* _tmp_2 = x_2; +lean_object* _tmp_9 = x_20; +x_2 = _tmp_1; +x_3 = _tmp_2; +x_10 = _tmp_9; +} +goto _start; } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; -x_48 = lean_ctor_get(x_18, 1); -lean_inc(x_48); -lean_dec(x_18); -lean_inc(x_15); -x_49 = lean_array_to_list(x_15); -x_50 = lean_box(0); -x_51 = l_List_mapTR_loop___at_Lean_Meta_Match_mkMatcher___spec__6(x_49, x_50); -x_52 = l_Lean_MessageData_ofList(x_51); -x_53 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__2; -x_54 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_54, 0, x_53); -lean_ctor_set(x_54, 1, x_52); -x_55 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__4; -x_56 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_56, 0, x_54); -lean_ctor_set(x_56, 1, x_55); -lean_inc(x_2); -x_57 = l_Lean_MessageData_ofLevel(x_2); -x_58 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_58, 0, x_56); -lean_ctor_set(x_58, 1, x_57); -x_59 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__6; -x_60 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_60, 0, x_58); -lean_ctor_set(x_60, 1, x_59); -lean_inc(x_3); -x_61 = l___private_Init_Data_Repr_0__Nat_reprFast(x_3); -x_62 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_62, 0, x_61); -x_63 = l_Lean_MessageData_ofFormat(x_62); -x_64 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_64, 0, x_60); -lean_ctor_set(x_64, 1, x_63); -x_65 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5; -x_66 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_66, 0, x_64); -lean_ctor_set(x_66, 1, x_65); -x_67 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_17, x_66, x_7, x_8, x_9, x_10, x_11, x_12, x_48); -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 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__1(x_4, x_5, x_15, x_3, x_2, x_68, x_7, x_8, x_9, x_10, x_11, x_12, x_69); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_68); -lean_dec(x_2); -lean_dec(x_3); -return x_70; +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_2, 1); +x_23 = lean_ctor_get(x_14, 0); +x_24 = lean_ctor_get(x_14, 1); +lean_inc(x_24); +lean_inc(x_23); +lean_dec(x_14); +lean_inc(x_1); +x_25 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27(x_1, x_24, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_26 = lean_ctor_get(x_25, 0); +lean_inc(x_26); +x_27 = lean_ctor_get(x_25, 1); +lean_inc(x_27); +lean_dec(x_25); +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_23); +lean_ctor_set(x_28, 1, x_26); +lean_ctor_set(x_2, 1, x_3); +lean_ctor_set(x_2, 0, x_28); +{ +lean_object* _tmp_1 = x_22; +lean_object* _tmp_2 = x_2; +lean_object* _tmp_9 = x_27; +x_2 = _tmp_1; +x_3 = _tmp_2; +x_10 = _tmp_9; } +goto _start; } } else { -uint8_t x_71; -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_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_30 = lean_ctor_get(x_2, 0); +x_31 = lean_ctor_get(x_2, 1); +lean_inc(x_31); +lean_inc(x_30); lean_dec(x_2); -x_71 = !lean_is_exclusive(x_14); -if (x_71 == 0) -{ -return x_14; -} -else -{ -lean_object* x_72; lean_object* x_73; lean_object* x_74; -x_72 = lean_ctor_get(x_14, 0); -x_73 = lean_ctor_get(x_14, 1); -lean_inc(x_73); -lean_inc(x_72); -lean_dec(x_14); -x_74 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_74, 0, x_72); -lean_ctor_set(x_74, 1, x_73); -return x_74; -} -} +x_32 = lean_ctor_get(x_30, 0); +lean_inc(x_32); +x_33 = lean_ctor_get(x_30, 1); +lean_inc(x_33); +if (lean_is_exclusive(x_30)) { + lean_ctor_release(x_30, 0); + lean_ctor_release(x_30, 1); + x_34 = x_30; +} else { + lean_dec_ref(x_30); + x_34 = lean_box(0); } +lean_inc(x_1); +x_35 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27(x_1, x_33, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +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); +if (lean_is_scalar(x_34)) { + x_38 = lean_alloc_ctor(0, 2, 0); +} else { + x_38 = x_34; } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("failed to compute resulting universe level of inductive datatype, provide universe explicitly: ", 95, 95); -return x_1; +lean_ctor_set(x_38, 0, x_32); +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_2 = x_31; +x_3 = x_39; +x_10 = x_37; +goto _start; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_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_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam___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_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_11) == 0) -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); -x_13 = lean_ctor_get(x_11, 1); -lean_inc(x_13); -lean_dec(x_11); -x_14 = lean_unsigned_to_nat(0u); -x_15 = l_Lean_Level_getOffsetAux(x_12, x_14); -x_16 = l_Lean_Level_getLevelOffset(x_12); -lean_dec(x_12); -x_17 = l_Lean_Level_isMVar(x_16); -if (x_17 == 0) -{ -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; -lean_dec(x_15); -lean_dec(x_3); -lean_dec(x_2); -x_18 = l_Lean_MessageData_ofLevel(x_16); -x_19 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___closed__2; -x_20 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_20, 0, x_19); -lean_ctor_set(x_20, 1, x_18); -x_21 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5; -x_22 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_22, 0, x_20); -lean_ctor_set(x_22, 1, x_21); -x_23 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_22, x_4, x_5, x_6, x_7, x_8, x_9, x_13); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -x_24 = !lean_is_exclusive(x_23); -if (x_24 == 0) +if (lean_obj_tag(x_2) == 0) { -return x_23; +lean_object* x_11; lean_object* x_12; +lean_dec(x_1); +x_11 = l_List_reverse___rarg(x_3); +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; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_23, 0); -x_26 = lean_ctor_get(x_23, 1); -lean_inc(x_26); +uint8_t x_13; +x_13 = !lean_is_exclusive(x_2); +if (x_13 == 0) +{ +lean_object* x_14; uint8_t x_15; +x_14 = lean_ctor_get(x_2, 0); +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; +x_16 = lean_ctor_get(x_2, 1); +x_17 = lean_ctor_get(x_14, 1); +x_18 = lean_ctor_get(x_14, 2); +lean_inc(x_1); +x_19 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27(x_1, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_19, 1); +lean_inc(x_21); +lean_dec(x_19); +x_22 = lean_box(0); +lean_inc(x_1); +x_23 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam___spec__1(x_1, x_18, x_22, x_4, x_5, x_6, x_7, x_8, x_9, x_21); +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_23, 1); lean_inc(x_25); lean_dec(x_23); -x_27 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_26); -return x_27; +lean_ctor_set(x_14, 2, x_24); +lean_ctor_set(x_14, 1, x_20); +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_25; +x_2 = _tmp_1; +x_3 = _tmp_2; +x_10 = _tmp_9; } +goto _start; } else { -lean_object* x_28; lean_object* x_29; -x_28 = lean_box(0); -x_29 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2(x_1, x_16, x_15, x_2, x_3, x_28, x_4, x_5, x_6, x_7, x_8, x_9, x_13); -return x_29; +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_27 = lean_ctor_get(x_2, 1); +x_28 = lean_ctor_get(x_14, 0); +x_29 = lean_ctor_get(x_14, 1); +x_30 = lean_ctor_get(x_14, 2); +lean_inc(x_30); +lean_inc(x_29); +lean_inc(x_28); +lean_dec(x_14); +lean_inc(x_1); +x_31 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27(x_1, x_29, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +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_1); +x_35 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam___spec__1(x_1, x_30, x_34, x_4, x_5, x_6, x_7, x_8, x_9, x_33); +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(0, 3, 0); +lean_ctor_set(x_38, 0, x_28); +lean_ctor_set(x_38, 1, x_32); +lean_ctor_set(x_38, 2, x_36); +lean_ctor_set(x_2, 1, x_3); +lean_ctor_set(x_2, 0, x_38); +{ +lean_object* _tmp_1 = x_27; +lean_object* _tmp_2 = x_2; +lean_object* _tmp_9 = x_37; +x_2 = _tmp_1; +x_3 = _tmp_2; +x_10 = _tmp_9; +} +goto _start; } } else { -uint8_t x_30; -lean_dec(x_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_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_40 = lean_ctor_get(x_2, 0); +x_41 = lean_ctor_get(x_2, 1); +lean_inc(x_41); +lean_inc(x_40); lean_dec(x_2); -x_30 = !lean_is_exclusive(x_11); -if (x_30 == 0) -{ -return x_11; +x_42 = lean_ctor_get(x_40, 0); +lean_inc(x_42); +x_43 = lean_ctor_get(x_40, 1); +lean_inc(x_43); +x_44 = lean_ctor_get(x_40, 2); +lean_inc(x_44); +if (lean_is_exclusive(x_40)) { + lean_ctor_release(x_40, 0); + lean_ctor_release(x_40, 1); + lean_ctor_release(x_40, 2); + x_45 = x_40; +} else { + lean_dec_ref(x_40); + x_45 = lean_box(0); } -else -{ -lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_31 = lean_ctor_get(x_11, 0); -x_32 = lean_ctor_get(x_11, 1); -lean_inc(x_32); -lean_inc(x_31); -lean_dec(x_11); -x_33 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_33, 0, x_31); -lean_ctor_set(x_33, 1, x_32); -return x_33; +lean_inc(x_1); +x_46 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27(x_1, x_43, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +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_box(0); +lean_inc(x_1); +x_50 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam___spec__1(x_1, x_44, x_49, x_4, x_5, x_6, x_7, x_8, x_9, x_48); +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); +if (lean_is_scalar(x_45)) { + x_53 = lean_alloc_ctor(0, 3, 0); +} else { + x_53 = x_45; } +lean_ctor_set(x_53, 0, x_42); +lean_ctor_set(x_53, 1, x_47); +lean_ctor_set(x_53, 2, x_51); +x_54 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_54, 0, x_53); +lean_ctor_set(x_54, 1, x_3); +x_2 = x_41; +x_3 = x_54; +x_10 = x_52; +goto _start; } } } -LEAN_EXPORT lean_object* l_Lean_assignLevelMVar___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___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_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_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) { _start: { -lean_object* x_10; -x_10 = l_Lean_assignLevelMVar___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_object* x_10; lean_object* x_11; +x_10 = lean_box(0); +x_11 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam___spec__2(x_2, 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_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam___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_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam___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); -return x_10; +return x_11; } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam___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_10; -x_10 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_object* x_11; +x_11 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam___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); -return x_10; +return x_11; } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___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_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_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) { _start: { lean_object* x_10; -x_10 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_10 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam(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); @@ -16561,1889 +17358,1877 @@ lean_dec(x_3); return x_10; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_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_mkResultUniverse(lean_object* x_1, lean_object* x_2, uint8_t x_3) { _start: { -lean_object* x_14; -x_14 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_8); -lean_dec(x_7); +uint8_t x_4; +x_4 = l_Array_isEmpty___rarg(x_1); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; +x_5 = lean_array_to_list(x_1); +x_6 = l_Lean_Level_mkNaryMax(x_5); +x_7 = lean_unsigned_to_nat(0u); +x_8 = lean_nat_dec_eq(x_2, x_7); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = l_Lean_Level_normalize(x_6); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -return x_14; -} +return x_9; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { -_start: +else { -lean_object* x_14; -x_14 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___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_6); -lean_dec(x_1); +uint8_t x_10; +x_10 = l_Lean_Level_isZero(x_6); +if (x_10 == 0) +{ +uint8_t x_11; +x_11 = l_Lean_Level_isNeverZero(x_6); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = l_Lean_levelOne; +x_13 = l_Lean_Level_max___override(x_6, x_12); +x_14 = l_Lean_Level_normalize(x_13); +lean_dec(x_13); return x_14; } -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: +else { -lean_object* x_11; -x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse(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_15; +x_15 = l_Lean_Level_normalize(x_6); +lean_dec(x_6); +return x_15; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("bootstrap", 9, 9); -return x_1; +lean_object* x_16; +x_16 = l_Lean_Level_normalize(x_6); +lean_dec(x_6); +return x_16; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__2() { -_start: +} +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("inductiveCheckResultingUniverse", 31, 31); -return x_1; +lean_object* x_17; uint8_t x_18; +x_17 = lean_unsigned_to_nat(0u); +x_18 = lean_nat_dec_eq(x_2, x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_array_to_list(x_1); +x_20 = l_Lean_Level_mkNaryMax(x_19); +x_21 = l_Lean_Level_normalize(x_20); +lean_dec(x_20); +return x_21; } +else +{ +lean_dec(x_1); +if (x_3 == 0) +{ +lean_object* x_22; +x_22 = l_Lean_levelOne; +return x_22; } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__3() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__1; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__2; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; +lean_object* x_23; +x_23 = l_Lean_levelZero; +return x_23; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("by default the `inductive`/`structure` commands report an error if the resulting universe is not zero, but may be zero for some universe parameters. Reason: unless this type is a subsingleton, it is hardly what the user wants since it can only eliminate into `Prop`. In the `Init` package, we define subsingletons, and we use this option to disable the check. This option may be deleted in the future after we improve the validator", 431, 431); -return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__5() { +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkResultUniverse___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _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_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__1; -x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__4; -x_4 = lean_box(x_1); -x_5 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_5, 0, x_4); -lean_ctor_set(x_5, 1, x_2); -lean_ctor_set(x_5, 2, x_3); +uint8_t x_4; lean_object* x_5; +x_4 = lean_unbox(x_3); +lean_dec(x_3); +x_5 = l_Lean_Elab_Command_mkResultUniverse(x_1, x_2, x_4); +lean_dec(x_2); return x_5; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__6() { +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Command_accLevel_go___spec__2(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_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_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__1; -x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__7; -x_4 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__1; -x_5 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__2; -x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); -return x_6; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063_(lean_object* x_1) { -_start: +uint8_t x_5; +x_5 = lean_usize_dec_eq(x_3, x_4); +if (x_5 == 0) { -lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__3; -x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__5; -x_4 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__6; -x_5 = l_Lean_Option_register___at_Lean_Elab_initFn____x40_Lean_Elab_AutoBound___hyg_6____spec__1(x_2, x_3, x_4, x_1); -return x_5; +lean_object* x_6; uint8_t x_7; +x_6 = lean_array_uget(x_2, x_3); +x_7 = lean_level_eq(x_6, x_1); +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; } -static lean_object* _init_l_Lean_Elab_Command_checkResultingUniverse___closed__1() { -_start: +} +else { -lean_object* x_1; -x_1 = l_Lean_Elab_Command_bootstrap_inductiveCheckResultingUniverse; -return x_1; +uint8_t x_12; +x_12 = 0; +return x_12; } } -static lean_object* _init_l_Lean_Elab_Command_checkResultingUniverse___closed__2() { +} +LEAN_EXPORT uint8_t l_Array_contains___at_Lean_Elab_Command_accLevel_go___spec__1(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("invalid universe polymorphic type, the resultant universe is not Prop (i.e., 0), but it may be Prop for some parameter values (solution: use 'u+1' or 'max 1 u')", 160, 160); -return x_1; +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 +{ +size_t x_7; size_t x_8; uint8_t x_9; +x_7 = 0; +x_8 = lean_usize_of_nat(x_3); +lean_dec(x_3); +x_9 = l_Array_anyMUnsafe_any___at_Lean_Elab_Command_accLevel_go___spec__2(x_2, x_1, x_7, x_8); +return x_9; } -static lean_object* _init_l_Lean_Elab_Command_checkResultingUniverse___closed__3() { +} +} +static lean_object* _init_l_Lean_Elab_Command_accLevel_go___closed__1() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_checkResultingUniverse___closed__2; -x_2 = l_Lean_stringToMessageData(x_1); +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_Elab_Command_checkResultingUniverse(lean_object* x_1, lean_object* x_2, lean_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_Command_accLevel_go(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_9; lean_object* x_10; uint8_t x_11; -x_9 = lean_ctor_get(x_6, 2); -x_10 = l_Lean_Elab_Command_checkResultingUniverse___closed__1; -x_11 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_9, x_10); -if (x_11 == 0) +lean_object* x_5; +switch (lean_obj_tag(x_2)) { +case 0: { -lean_object* x_12; lean_object* x_13; +lean_object* x_20; lean_object* x_21; +lean_dec(x_3); +x_20 = l_Lean_Elab_Command_accLevel_go___closed__1; +x_21 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_21, 0, x_20); +lean_ctor_set(x_21, 1, x_4); +return x_21; +} +case 1: +{ +lean_object* x_22; lean_object* x_23; uint8_t x_24; +x_22 = lean_ctor_get(x_2, 0); +lean_inc(x_22); +x_23 = lean_unsigned_to_nat(0u); +x_24 = lean_nat_dec_eq(x_3, x_23); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; lean_dec(x_2); -lean_dec(x_1); -x_12 = lean_box(0); -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_12); -lean_ctor_set(x_13, 1, x_8); -return x_13; +x_25 = lean_unsigned_to_nat(1u); +x_26 = lean_nat_sub(x_3, x_25); +lean_dec(x_3); +x_2 = x_22; +x_3 = x_26; +goto _start; } else { -lean_object* x_14; uint8_t x_15; -x_14 = l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_shouldInferResultUniverse___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -x_15 = !lean_is_exclusive(x_14); -if (x_15 == 0) +uint8_t x_28; +lean_dec(x_22); +lean_dec(x_3); +x_28 = lean_level_eq(x_2, x_1); +if (x_28 == 0) { -lean_object* x_16; lean_object* x_17; uint8_t x_18; -x_16 = lean_ctor_get(x_14, 0); -x_17 = lean_ctor_get(x_14, 1); -x_18 = l_Lean_Level_isZero(x_16); -if (x_18 == 0) +uint8_t x_29; +x_29 = l_Lean_Level_occurs(x_1, x_2); +if (x_29 == 0) { -uint8_t x_19; -x_19 = l_Lean_Level_isNeverZero(x_16); -if (x_19 == 0) +uint8_t x_30; +x_30 = l_Array_contains___at_Lean_Elab_Command_accLevel_go___spec__1(x_4, x_2); +if (x_30 == 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_free_object(x_14); -x_20 = l_Lean_MessageData_ofLevel(x_16); -x_21 = l_Lean_indentD(x_20); -x_22 = l_Lean_Elab_Command_checkResultingUniverse___closed__3; -x_23 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_23, 0, x_22); -lean_ctor_set(x_23, 1, x_21); -x_24 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5; -x_25 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_25, 0, x_23); -lean_ctor_set(x_25, 1, x_24); -x_26 = l_Lean_throwError___at_Lean_Elab_Term_throwErrorIfErrors___spec__1(x_25, x_2, x_3, x_4, x_5, x_6, x_7, x_17); -return x_26; +lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_31 = lean_array_push(x_4, x_2); +x_32 = l_Lean_Elab_Command_accLevel_go___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); +return x_33; } else { -lean_object* x_27; -lean_dec(x_16); +lean_object* x_34; lean_object* x_35; lean_dec(x_2); -x_27 = lean_box(0); -lean_ctor_set(x_14, 0, x_27); -return x_14; +x_34 = l_Lean_Elab_Command_accLevel_go___closed__1; +x_35 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_35, 0, x_34); +lean_ctor_set(x_35, 1, x_4); +return x_35; } } else { -lean_object* x_28; -lean_dec(x_16); +lean_object* x_36; lean_object* x_37; lean_dec(x_2); -x_28 = lean_box(0); -lean_ctor_set(x_14, 0, x_28); -return x_14; +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_4); +return x_37; } } else { -lean_object* x_29; lean_object* x_30; uint8_t 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 = l_Lean_Level_isZero(x_29); -if (x_31 == 0) +lean_object* x_38; lean_object* x_39; +lean_dec(x_2); +x_38 = l_Lean_Elab_Command_accLevel_go___closed__1; +x_39 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_39, 0, x_38); +lean_ctor_set(x_39, 1, x_4); +return x_39; +} +} +} +case 4: { -uint8_t x_32; -x_32 = l_Lean_Level_isNeverZero(x_29); -if (x_32 == 0) +lean_object* x_40; uint8_t x_41; +x_40 = lean_unsigned_to_nat(0u); +x_41 = lean_nat_dec_eq(x_3, x_40); +if (x_41 == 0) { -lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_33 = l_Lean_MessageData_ofLevel(x_29); -x_34 = l_Lean_indentD(x_33); -x_35 = l_Lean_Elab_Command_checkResultingUniverse___closed__3; -x_36 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_36, 0, x_35); -lean_ctor_set(x_36, 1, x_34); -x_37 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5; -x_38 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -x_39 = l_Lean_throwError___at_Lean_Elab_Term_throwErrorIfErrors___spec__1(x_38, x_2, x_3, x_4, x_5, x_6, x_7, x_30); -return x_39; +lean_object* x_42; +x_42 = lean_box(0); +x_5 = x_42; +goto block_19; } else { -lean_object* x_40; lean_object* x_41; -lean_dec(x_29); -lean_dec(x_2); -x_40 = lean_box(0); -x_41 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_41, 0, x_40); -lean_ctor_set(x_41, 1, x_30); -return x_41; -} +uint8_t x_43; +x_43 = lean_level_eq(x_2, x_1); +if (x_43 == 0) +{ +lean_object* x_44; +x_44 = lean_box(0); +x_5 = x_44; +goto block_19; } else { -lean_object* x_42; lean_object* x_43; -lean_dec(x_29); +lean_object* x_45; lean_object* x_46; +lean_dec(x_3); lean_dec(x_2); -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_30); -return x_43; +x_45 = l_Lean_Elab_Command_accLevel_go___closed__1; +x_46 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_46, 0, x_45); +lean_ctor_set(x_46, 1, x_4); +return x_46; } } } +case 5: +{ +lean_object* x_47; uint8_t x_48; +x_47 = lean_unsigned_to_nat(0u); +x_48 = lean_nat_dec_eq(x_3, x_47); +if (x_48 == 0) +{ +lean_object* x_49; +x_49 = lean_box(0); +x_5 = x_49; +goto block_19; } +else +{ +uint8_t x_50; +x_50 = lean_level_eq(x_2, x_1); +if (x_50 == 0) +{ +lean_object* x_51; +x_51 = lean_box(0); +x_5 = x_51; +goto block_19; } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkResultingUniverse___boxed(lean_object* x_1, lean_object* x_2, lean_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_Command_checkResultingUniverse(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_object* x_52; lean_object* x_53; lean_dec(x_3); -return x_9; +lean_dec(x_2); +x_52 = l_Lean_Elab_Command_accLevel_go___closed__1; +x_53 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_53, 0, x_52); +lean_ctor_set(x_53, 1, x_4); +return x_53; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { -_start: +} +default: { -uint8_t x_15; -x_15 = lean_usize_dec_lt(x_6, x_5); -if (x_15 == 0) +lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_54 = lean_ctor_get(x_2, 0); +lean_inc(x_54); +x_55 = lean_ctor_get(x_2, 1); +lean_inc(x_55); +lean_dec(x_2); +lean_inc(x_3); +x_56 = l_Lean_Elab_Command_accLevel_go(x_1, x_54, x_3, x_4); +x_57 = lean_ctor_get(x_56, 0); +lean_inc(x_57); +if (lean_obj_tag(x_57) == 0) { -lean_object* 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); +uint8_t x_58; +lean_dec(x_55); lean_dec(x_3); -lean_dec(x_2); -x_16 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_16, 0, x_7); -lean_ctor_set(x_16, 1, x_14); -return x_16; +x_58 = !lean_is_exclusive(x_56); +if (x_58 == 0) +{ +lean_object* x_59; lean_object* x_60; +x_59 = lean_ctor_get(x_56, 0); +lean_dec(x_59); +x_60 = lean_box(0); +lean_ctor_set(x_56, 0, x_60); +return x_56; } else { -lean_object* x_17; lean_object* x_18; uint8_t x_19; -lean_dec(x_7); -x_17 = lean_array_uget(x_4, x_6); -x_18 = lean_ctor_get(x_17, 2); -lean_inc(x_18); -x_19 = lean_name_eq(x_18, x_1); -lean_dec(x_18); -if (x_19 == 0) -{ -size_t x_20; size_t x_21; -lean_dec(x_17); -x_20 = 1; -x_21 = lean_usize_add(x_6, x_20); -lean_inc(x_3); -{ -size_t _tmp_5 = x_21; -lean_object* _tmp_6 = x_3; -x_6 = _tmp_5; -x_7 = _tmp_6; +lean_object* x_61; lean_object* x_62; lean_object* x_63; +x_61 = lean_ctor_get(x_56, 1); +lean_inc(x_61); +lean_dec(x_56); +x_62 = lean_box(0); +x_63 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_63, 0, x_62); +lean_ctor_set(x_63, 1, x_61); +return x_63; } -goto _start; } else { -lean_object* x_23; uint8_t x_24; +lean_object* x_64; +lean_dec(x_57); +x_64 = lean_ctor_get(x_56, 1); +lean_inc(x_64); +lean_dec(x_56); +x_2 = x_55; +x_4 = x_64; +goto _start; +} +} +} +block_19: +{ +uint8_t x_6; +lean_dec(x_5); +x_6 = l_Lean_Level_occurs(x_1, x_2); +if (x_6 == 0) +{ +lean_object* x_7; uint8_t x_8; +x_7 = lean_unsigned_to_nat(0u); +x_8 = lean_nat_dec_lt(x_7, x_3); lean_dec(x_3); -x_23 = lean_ctor_get(x_17, 0); -lean_inc(x_23); -lean_dec(x_17); -x_24 = !lean_is_exclusive(x_12); -if (x_24 == 0) +if (x_8 == 0) { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_12, 5); -x_26 = l_Lean_replaceRef(x_23, x_25); -lean_dec(x_25); -lean_dec(x_23); -lean_ctor_set(x_12, 5, x_26); -x_27 = lean_apply_7(x_2, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -if (lean_obj_tag(x_27) == 0) +uint8_t x_9; +x_9 = l_Array_contains___at_Lean_Elab_Command_accLevel_go___spec__1(x_4, x_2); +if (x_9 == 0) { -uint8_t x_28; -x_28 = !lean_is_exclusive(x_27); -if (x_28 == 0) +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_array_push(x_4, x_2); +x_11 = l_Lean_Elab_Command_accLevel_go___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); +return x_12; +} +else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_29 = lean_ctor_get(x_27, 0); -x_30 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_30, 0, x_29); -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_27, 0, x_32); -return x_27; +lean_object* x_13; lean_object* x_14; +lean_dec(x_2); +x_13 = l_Lean_Elab_Command_accLevel_go___closed__1; +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_13); +lean_ctor_set(x_14, 1, x_4); +return x_14; +} } 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; -x_33 = lean_ctor_get(x_27, 0); -x_34 = lean_ctor_get(x_27, 1); -lean_inc(x_34); -lean_inc(x_33); -lean_dec(x_27); -x_35 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_35, 0, x_33); -x_36 = lean_box(0); -x_37 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -x_38 = lean_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_object* x_15; lean_object* x_16; +lean_dec(x_2); +x_15 = lean_box(0); +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_16, 1, x_4); +return x_16; } } else { -uint8_t x_39; -x_39 = !lean_is_exclusive(x_27); -if (x_39 == 0) +lean_object* x_17; lean_object* x_18; +lean_dec(x_3); +lean_dec(x_2); +x_17 = lean_box(0); +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set(x_18, 1, x_4); +return x_18; +} +} +} +} +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Command_accLevel_go___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: { -return x_27; +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_Command_accLevel_go___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; } -else +} +LEAN_EXPORT lean_object* l_Array_contains___at_Lean_Elab_Command_accLevel_go___spec__1___boxed(lean_object* x_1, lean_object* x_2) { +_start: { -lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_40 = lean_ctor_get(x_27, 0); -x_41 = lean_ctor_get(x_27, 1); -lean_inc(x_41); -lean_inc(x_40); -lean_dec(x_27); -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; +uint8_t x_3; lean_object* x_4; +x_3 = l_Array_contains___at_Lean_Elab_Command_accLevel_go___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_Lean_Elab_Command_accLevel_go___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Lean_Elab_Command_accLevel_go(x_1, x_2, x_3, x_4); +lean_dec(x_1); +return x_5; +} } -else +LEAN_EXPORT lean_object* l_Lean_Elab_Command_accLevel(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: { -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; uint8_t x_54; lean_object* x_55; uint8_t x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; -x_43 = lean_ctor_get(x_12, 0); -x_44 = lean_ctor_get(x_12, 1); -x_45 = lean_ctor_get(x_12, 2); -x_46 = lean_ctor_get(x_12, 3); -x_47 = lean_ctor_get(x_12, 4); -x_48 = lean_ctor_get(x_12, 5); -x_49 = lean_ctor_get(x_12, 6); -x_50 = lean_ctor_get(x_12, 7); -x_51 = lean_ctor_get(x_12, 8); -x_52 = lean_ctor_get(x_12, 9); -x_53 = lean_ctor_get(x_12, 10); -x_54 = lean_ctor_get_uint8(x_12, sizeof(void*)*12); -x_55 = lean_ctor_get(x_12, 11); -x_56 = lean_ctor_get_uint8(x_12, sizeof(void*)*12 + 1); -lean_inc(x_55); -lean_inc(x_53); -lean_inc(x_52); -lean_inc(x_51); -lean_inc(x_50); -lean_inc(x_49); -lean_inc(x_48); -lean_inc(x_47); -lean_inc(x_46); -lean_inc(x_45); -lean_inc(x_44); -lean_inc(x_43); -lean_dec(x_12); -x_57 = l_Lean_replaceRef(x_23, x_48); -lean_dec(x_48); -lean_dec(x_23); -x_58 = lean_alloc_ctor(0, 12, 2); -lean_ctor_set(x_58, 0, x_43); -lean_ctor_set(x_58, 1, x_44); -lean_ctor_set(x_58, 2, x_45); -lean_ctor_set(x_58, 3, x_46); -lean_ctor_set(x_58, 4, x_47); -lean_ctor_set(x_58, 5, x_57); -lean_ctor_set(x_58, 6, x_49); -lean_ctor_set(x_58, 7, x_50); -lean_ctor_set(x_58, 8, x_51); -lean_ctor_set(x_58, 9, x_52); -lean_ctor_set(x_58, 10, x_53); -lean_ctor_set(x_58, 11, x_55); -lean_ctor_set_uint8(x_58, sizeof(void*)*12, x_54); -lean_ctor_set_uint8(x_58, sizeof(void*)*12 + 1, x_56); -x_59 = lean_apply_7(x_2, x_8, x_9, x_10, x_11, x_58, x_13, x_14); -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; lean_object* x_65; lean_object* x_66; -x_60 = lean_ctor_get(x_59, 0); -lean_inc(x_60); -x_61 = lean_ctor_get(x_59, 1); -lean_inc(x_61); -if (lean_is_exclusive(x_59)) { - lean_ctor_release(x_59, 0); - lean_ctor_release(x_59, 1); - x_62 = x_59; -} else { - lean_dec_ref(x_59); - x_62 = lean_box(0); -} -x_63 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_63, 0, x_60); -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); -if (lean_is_scalar(x_62)) { - x_66 = lean_alloc_ctor(0, 2, 0); -} else { - x_66 = x_62; +lean_object* x_5; +x_5 = l_Lean_Elab_Command_accLevel_go(x_2, x_1, x_3, x_4); +return x_5; } -lean_ctor_set(x_66, 0, x_65); -lean_ctor_set(x_66, 1, x_61); -return x_66; } -else +LEAN_EXPORT lean_object* l_Lean_Elab_Command_accLevel___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: { -lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; -x_67 = lean_ctor_get(x_59, 0); -lean_inc(x_67); -x_68 = lean_ctor_get(x_59, 1); -lean_inc(x_68); -if (lean_is_exclusive(x_59)) { - lean_ctor_release(x_59, 0); - lean_ctor_release(x_59, 1); - x_69 = x_59; -} else { - lean_dec_ref(x_59); - x_69 = lean_box(0); -} -if (lean_is_scalar(x_69)) { - x_70 = lean_alloc_ctor(1, 2, 0); -} else { - x_70 = x_69; -} -lean_ctor_set(x_70, 0, x_67); -lean_ctor_set(x_70, 1, x_68); -return x_70; -} -} -} -} +lean_object* x_5; +x_5 = l_Lean_Elab_Command_accLevel(x_1, x_2, x_3, x_4); +lean_dec(x_2); +return x_5; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_accLevelAtCtor___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -uint8_t x_15; -x_15 = lean_usize_dec_lt(x_6, x_5); -if (x_15 == 0) -{ -lean_object* x_16; -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; 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_st_ref_get(x_6, 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); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_3); -lean_dec(x_2); -x_16 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_16, 0, x_7); -lean_ctor_set(x_16, 1, x_14); -return x_16; -} -else -{ -lean_object* x_17; lean_object* x_18; size_t x_19; size_t x_20; lean_object* x_21; -lean_dec(x_7); -x_17 = lean_array_uget(x_4, x_6); -x_18 = lean_ctor_get(x_17, 8); +x_13 = lean_ctor_get(x_11, 0); +lean_inc(x_13); +lean_dec(x_11); +x_14 = lean_instantiate_level_mvars(x_13, x_1); +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_take(x_6, x_12); +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_array_size(x_18); -x_20 = 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); -lean_inc_n(x_3, 2); -lean_inc(x_2); -x_21 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___spec__2(x_1, x_2, x_3, x_18, x_19, x_20, x_3, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -lean_dec(x_18); -if (lean_obj_tag(x_21) == 0) -{ -lean_object* x_22; lean_object* x_23; -x_22 = lean_ctor_get(x_21, 0); -lean_inc(x_22); -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -lean_dec(x_22); -if (lean_obj_tag(x_23) == 0) +x_20 = !lean_is_exclusive(x_18); +if (x_20 == 0) { -lean_object* x_24; size_t x_25; size_t x_26; -x_24 = lean_ctor_get(x_21, 1); -lean_inc(x_24); +lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_21 = lean_ctor_get(x_18, 0); lean_dec(x_21); -x_25 = 1; -x_26 = lean_usize_add(x_6, x_25); -lean_inc(x_3); -{ -size_t _tmp_5 = x_26; -lean_object* _tmp_6 = x_3; -lean_object* _tmp_13 = x_24; -x_6 = _tmp_5; -x_7 = _tmp_6; -x_14 = _tmp_13; -} -goto _start; -} -else -{ -uint8_t x_28; -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_3); -lean_dec(x_2); -x_28 = !lean_is_exclusive(x_21); -if (x_28 == 0) -{ -lean_object* x_29; uint8_t x_30; -x_29 = lean_ctor_get(x_21, 0); -lean_dec(x_29); -x_30 = !lean_is_exclusive(x_23); -if (x_30 == 0) +lean_ctor_set(x_18, 0, x_15); +x_22 = lean_st_ref_set(x_6, x_18, x_19); +x_23 = !lean_is_exclusive(x_22); +if (x_23 == 0) { -lean_object* x_31; lean_object* x_32; -x_31 = lean_box(0); -x_32 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_32, 0, x_23); -lean_ctor_set(x_32, 1, x_31); -lean_ctor_set(x_21, 0, x_32); -return x_21; +lean_object* x_24; +x_24 = lean_ctor_get(x_22, 0); +lean_dec(x_24); +lean_ctor_set(x_22, 0, x_16); +return x_22; } 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_box(0); -x_36 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_36, 0, x_34); -lean_ctor_set(x_36, 1, x_35); -lean_ctor_set(x_21, 0, x_36); -return x_21; +lean_object* x_25; lean_object* x_26; +x_25 = lean_ctor_get(x_22, 1); +lean_inc(x_25); +lean_dec(x_22); +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_16); +lean_ctor_set(x_26, 1, x_25); +return x_26; } } else { -lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_37 = lean_ctor_get(x_21, 1); -lean_inc(x_37); -lean_dec(x_21); -x_38 = lean_ctor_get(x_23, 0); -lean_inc(x_38); -if (lean_is_exclusive(x_23)) { - lean_ctor_release(x_23, 0); - x_39 = x_23; +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_27 = lean_ctor_get(x_18, 1); +x_28 = lean_ctor_get(x_18, 2); +x_29 = lean_ctor_get(x_18, 3); +x_30 = lean_ctor_get(x_18, 4); +lean_inc(x_30); +lean_inc(x_29); +lean_inc(x_28); +lean_inc(x_27); +lean_dec(x_18); +x_31 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_31, 0, x_15); +lean_ctor_set(x_31, 1, x_27); +lean_ctor_set(x_31, 2, x_28); +lean_ctor_set(x_31, 3, x_29); +lean_ctor_set(x_31, 4, x_30); +x_32 = lean_st_ref_set(x_6, x_31, x_19); +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_23); - x_39 = lean_box(0); + lean_dec_ref(x_32); + x_34 = lean_box(0); } -if (lean_is_scalar(x_39)) { - x_40 = lean_alloc_ctor(1, 1, 0); +if (lean_is_scalar(x_34)) { + x_35 = lean_alloc_ctor(0, 2, 0); } else { - x_40 = x_39; + x_35 = x_34; } -lean_ctor_set(x_40, 0, x_38); -x_41 = lean_box(0); -x_42 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_42, 0, x_40); -lean_ctor_set(x_42, 1, x_41); -x_43 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_43, 0, x_42); -lean_ctor_set(x_43, 1, x_37); -return x_43; +lean_ctor_set(x_35, 0, x_16); +lean_ctor_set(x_35, 1, x_33); +return x_35; } } } -else +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_accLevelAtCtor___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: { -uint8_t x_44; -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_3); -lean_dec(x_2); -x_44 = !lean_is_exclusive(x_21); -if (x_44 == 0) +lean_object* x_10; lean_object* x_11; uint8_t x_12; +x_10 = lean_ctor_get(x_7, 5); +x_11 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_1, x_5, x_6, x_7, x_8, x_9); +x_12 = !lean_is_exclusive(x_11); +if (x_12 == 0) { -return x_21; +lean_object* x_13; lean_object* x_14; +x_13 = lean_ctor_get(x_11, 0); +lean_inc(x_10); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_10); +lean_ctor_set(x_14, 1, x_13); +lean_ctor_set_tag(x_11, 1); +lean_ctor_set(x_11, 0, x_14); +return x_11; } else { -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_21, 0); -x_46 = lean_ctor_get(x_21, 1); -lean_inc(x_46); -lean_inc(x_45); -lean_dec(x_21); -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_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); +lean_inc(x_10); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_10); +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_16); +return x_18; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_withCtorRef___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_accLevelAtCtor___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_10; -x_10 = lean_apply_7(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_10; +lean_object* x_11; +x_11 = l_Lean_throwError___at_Lean_Elab_Command_accLevelAtCtor___spec__2(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_11; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_withCtorRef___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__1() { _start: { -size_t x_11; size_t x_12; lean_object* x_13; lean_object* x_14; -x_11 = lean_array_size(x_1); -x_12 = 0; -x_13 = l_Lean_Elab_Command_withCtorRef___rarg___closed__1; -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -x_14 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___spec__3(x_2, x_3, x_13, x_1, x_11, x_12, x_13, 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; -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_17; lean_object* x_18; -x_17 = lean_ctor_get(x_14, 1); -lean_inc(x_17); -lean_dec(x_14); -x_18 = lean_apply_7(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_17); -return x_18; -} -else -{ -uint8_t x_19; -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_19 = !lean_is_exclusive(x_14); -if (x_19 == 0) -{ -lean_object* x_20; lean_object* x_21; -x_20 = lean_ctor_get(x_14, 0); -lean_dec(x_20); -x_21 = lean_ctor_get(x_16, 0); -lean_inc(x_21); -lean_dec(x_16); -lean_ctor_set(x_14, 0, x_21); -return x_14; -} -else -{ -lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_22 = lean_ctor_get(x_14, 1); -lean_inc(x_22); -lean_dec(x_14); -x_23 = lean_ctor_get(x_16, 0); -lean_inc(x_23); -lean_dec(x_16); -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_1; +x_1 = lean_mk_string_unchecked(" has type", 9, 9); +return x_1; } -else -{ -uint8_t x_25; -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_25 = !lean_is_exclusive(x_14); -if (x_25 == 0) -{ -return x_14; } -else +static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__2() { +_start: { -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_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; -} -} +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1___closed__1() { +static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__3() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("\nat universe level", 18, 18); +x_1 = lean_mk_string_unchecked("\ninductive type resulting type", 30, 30); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1___closed__2() { +static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1___closed__1; +x_1 = l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__3; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1___closed__3() { +static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__5() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("\nit must be smaller than or equal to the inductive datatype universe level", 74, 74); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Command_accLevelAtCtor___lambda__1___boxed), 10, 0); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1___closed__4() { +static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("\nrecall that Lean only infers the resulting universe level automatically when there is a unique solution for the universe level constraints, consider explicitly providing the inductive type resulting universe level", 214, 214); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__7() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1___closed__3; -x_2 = l_Lean_stringToMessageData(x_1); +x_1 = l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__6; +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_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___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) { +static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__8() { _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; lean_object* x_34; -x_15 = l_Lean_indentExpr(x_1); -x_16 = l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__2; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__7; +x_2 = l_Lean_MessageData_ofFormat(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_accLevelAtCtor___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; 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_15 = l_Lean_MessageData_ofExpr(x_1); +x_16 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; x_17 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_17, 0, x_16); lean_ctor_set(x_17, 1, x_15); -x_18 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5; +x_18 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___closed__6; x_19 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_19, 0, x_17); lean_ctor_set(x_19, 1, x_18); -x_20 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_20, 0, x_6); -lean_ctor_set(x_20, 1, x_19); -x_21 = l_Lean_MessageData_ofLevel(x_2); -x_22 = l_Lean_indentD(x_21); -x_23 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1___closed__2; -x_24 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_24, 0, x_23); -lean_ctor_set(x_24, 1, x_22); +x_20 = l_Lean_MessageData_ofExpr(x_2); +x_21 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_21, 0, x_19); +lean_ctor_set(x_21, 1, x_20); +x_22 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_22, 0, x_21); +lean_ctor_set(x_22, 1, x_16); +x_23 = l_Lean_indentD(x_22); +x_24 = l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__2; x_25 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_25, 0, x_24); -lean_ctor_set(x_25, 1, x_18); -x_26 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_26, 0, x_20); -lean_ctor_set(x_26, 1, x_25); -x_27 = l_Lean_MessageData_ofLevel(x_3); -x_28 = l_Lean_indentD(x_27); -x_29 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1___closed__4; -x_30 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_30, 0, x_29); -lean_ctor_set(x_30, 1, x_28); +lean_ctor_set(x_25, 1, x_23); +x_26 = l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__4; +x_27 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +lean_inc(x_4); +x_28 = l_Lean_Level_addOffsetAux(x_3, x_4); +x_29 = l_Lean_Expr_sort___override(x_28); +x_30 = l_Lean_indentExpr(x_29); x_31 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_31, 0, x_30); -lean_ctor_set(x_31, 1, x_18); +lean_ctor_set(x_31, 0, x_27); +lean_ctor_set(x_31, 1, x_30); x_32 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_32, 0, x_26); -lean_ctor_set(x_32, 1, x_31); -x_33 = lean_alloc_closure((void*)(l_Lean_throwError___at_Lean_Elab_Term_throwErrorIfErrors___spec__1___boxed), 8, 1); -lean_closure_set(x_33, 0, x_32); -x_34 = l_Lean_Elab_Command_withCtorRef___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___spec__1(x_4, x_5, x_33, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -return x_34; +lean_ctor_set(x_32, 0, x_31); +lean_ctor_set(x_32, 1, x_16); +x_33 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_33, 0, x_5); +lean_ctor_set(x_33, 1, x_32); +x_34 = l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__5; +x_35 = l_Lean_Level_isMVar(x_4); +lean_dec(x_4); +if (x_35 == 0) +{ +lean_object* x_36; lean_object* x_37; +x_36 = lean_box(0); +x_37 = lean_apply_10(x_34, x_33, x_36, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +return x_37; +} +else +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_38 = l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__8; +x_39 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_39, 0, x_33); +lean_ctor_set(x_39, 1, x_38); +x_40 = lean_box(0); +x_41 = lean_apply_10(x_34, x_39, x_40, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +return x_41; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___closed__1() { +} +static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("invalid universe level in constructor '", 39, 39); +x_1 = lean_mk_string_unchecked("failed to compute resulting universe level of inductive datatype, constructor '", 79, 79); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___closed__2() { +static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___closed__1; +x_1 = l_Lean_Elab_Command_accLevelAtCtor___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___closed__3() { +static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___closed__3() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("', parameter", 12, 12); +x_1 = lean_mk_string_unchecked("' has type", 10, 10); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___closed__4() { +static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___closed__3; +x_1 = l_Lean_Elab_Command_accLevelAtCtor___closed__3; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_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, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___closed__5() { _start: { -switch (lean_obj_tag(x_7)) { -case 1: +lean_object* x_1; +x_1 = lean_mk_string_unchecked("\nparameter", 10, 10); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___closed__6() { +_start: { -if (lean_obj_tag(x_8) == 1) +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_accLevelAtCtor___closed__5; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___closed__7() { +_start: { -lean_object* x_16; lean_object* x_17; -x_16 = lean_ctor_get(x_7, 0); -lean_inc(x_16); -lean_dec(x_7); -x_17 = lean_ctor_get(x_8, 0); -lean_inc(x_17); -lean_dec(x_8); -x_7 = x_16; -x_8 = x_17; -goto _start; +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" '", 2, 2); +return x_1; } -else +} +static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___closed__8() { +_start: { -uint8_t x_19; -lean_dec(x_8); -lean_dec(x_7); -x_19 = l_Lean_Level_geq(x_2, x_6); -if (x_19 == 0) +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_accLevelAtCtor___closed__7; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___closed__9() { +_start: { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_20 = lean_ctor_get(x_3, 0); -lean_inc(x_20); -lean_dec(x_3); -lean_inc(x_20); -x_21 = l_Lean_MessageData_ofName(x_20); -x_22 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___closed__2; -x_23 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_23, 0, x_22); -lean_ctor_set(x_23, 1, x_21); -x_24 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___closed__4; -x_25 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_25, 0, x_23); -lean_ctor_set(x_25, 1, x_24); +lean_object* x_1; +x_1 = lean_mk_string_unchecked("'", 1, 1); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Command_accLevelAtCtor___closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_accLevelAtCtor___closed__9; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_accLevelAtCtor(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, 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); -x_26 = l_Lean_Meta_getFVarLocalDecl(x_4, x_11, x_12, x_13, x_14, x_15); -if (lean_obj_tag(x_26) == 0) +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_2); +x_13 = lean_infer_type(x_2, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_13) == 0) { -lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; -x_27 = lean_ctor_get(x_26, 0); -lean_inc(x_27); -x_28 = lean_ctor_get(x_26, 1); -lean_inc(x_28); -lean_dec(x_26); -x_29 = l_Lean_LocalDecl_userName(x_27); -lean_dec(x_27); -x_30 = l_Lean_Name_hasMacroScopes(x_29); -lean_dec(x_29); -if (x_30 == 0) +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_13, 1); +lean_inc(x_15); +lean_dec(x_13); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_14); +x_16 = l_Lean_Meta_getLevel(x_14, x_8, x_9, x_10, x_11, x_15); +if (lean_obj_tag(x_16) == 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 = l_Lean_MessageData_ofExpr(x_4); -x_32 = l_Lean_Elab_Command_accLevelAtCtor___closed__8; -x_33 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_33, 0, x_32); -lean_ctor_set(x_33, 1, x_31); -x_34 = l_Lean_Elab_Command_accLevelAtCtor___closed__10; -x_35 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_35, 0, x_33); -lean_ctor_set(x_35, 1, x_34); -x_36 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_36, 0, x_25); -lean_ctor_set(x_36, 1, x_35); -x_37 = lean_box(0); -x_38 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1(x_5, x_6, x_2, x_1, x_20, x_36, x_37, x_9, x_10, x_11, x_12, x_13, x_14, x_28); -lean_dec(x_20); -return x_38; +lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +x_19 = l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_accLevelAtCtor___spec__1(x_17, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_18); +x_20 = !lean_is_exclusive(x_19); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; +x_21 = lean_ctor_get(x_19, 0); +x_22 = lean_ctor_get(x_19, 1); +x_23 = lean_st_ref_take(x_5, x_22); +x_24 = !lean_is_exclusive(x_23); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; +x_25 = lean_ctor_get(x_23, 0); +x_26 = lean_ctor_get(x_23, 1); +lean_inc(x_4); +x_27 = l_Lean_Elab_Command_accLevel_go(x_3, x_21, x_4, x_25); +x_28 = !lean_is_exclusive(x_27); +if (x_28 == 0) +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_27, 0); +x_30 = lean_ctor_get(x_27, 1); +x_31 = lean_st_ref_set(x_5, x_30, x_26); +if (lean_obj_tag(x_29) == 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); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_14); +x_33 = lean_infer_type(x_14, x_8, x_9, x_10, x_11, x_32); +if (lean_obj_tag(x_33) == 0) +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_34 = lean_ctor_get(x_33, 0); +lean_inc(x_34); +x_35 = lean_ctor_get(x_33, 1); +lean_inc(x_35); +lean_dec(x_33); +x_36 = lean_ctor_get(x_1, 0); +lean_inc(x_36); +x_37 = l_Lean_MessageData_ofName(x_36); +x_38 = l_Lean_Elab_Command_accLevelAtCtor___closed__2; +lean_ctor_set_tag(x_27, 7); +lean_ctor_set(x_27, 1, x_37); +lean_ctor_set(x_27, 0, x_38); +x_39 = l_Lean_Elab_Command_accLevelAtCtor___closed__4; +lean_ctor_set_tag(x_23, 7); +lean_ctor_set(x_23, 1, x_39); +lean_ctor_set(x_23, 0, x_27); +x_40 = lean_ctor_get(x_1, 1); +lean_inc(x_40); +lean_dec(x_1); +x_41 = l_Lean_indentExpr(x_40); +lean_ctor_set_tag(x_19, 7); +lean_ctor_set(x_19, 1, x_41); +lean_ctor_set(x_19, 0, x_23); +x_42 = l_Lean_Elab_Command_accLevelAtCtor___closed__6; +x_43 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_43, 0, x_19); +lean_ctor_set(x_43, 1, x_42); +lean_inc(x_8); +x_44 = l_Lean_Meta_getFVarLocalDecl(x_2, x_8, x_9, x_10, x_11, x_35); +if (lean_obj_tag(x_44) == 0) +{ +lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; +x_45 = lean_ctor_get(x_44, 0); +lean_inc(x_45); +x_46 = lean_ctor_get(x_44, 1); +lean_inc(x_46); +lean_dec(x_44); +x_47 = l_Lean_LocalDecl_userName(x_45); +lean_dec(x_45); +x_48 = l_Lean_Name_hasMacroScopes(x_47); +lean_dec(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; +x_49 = l_Lean_MessageData_ofExpr(x_2); +x_50 = l_Lean_Elab_Command_accLevelAtCtor___closed__8; +x_51 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_51, 0, x_50); +lean_ctor_set(x_51, 1, x_49); +x_52 = l_Lean_Elab_Command_accLevelAtCtor___closed__10; +x_53 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_53, 0, x_51); +lean_ctor_set(x_53, 1, x_52); +x_54 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_54, 0, x_43); +lean_ctor_set(x_54, 1, x_53); +x_55 = lean_box(0); +x_56 = l_Lean_Elab_Command_accLevelAtCtor___lambda__2(x_14, x_34, x_4, x_3, x_54, x_55, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_46); +return x_56; } else { -lean_object* x_39; lean_object* x_40; -lean_dec(x_4); -x_39 = lean_box(0); -x_40 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1(x_5, x_6, x_2, x_1, x_20, x_25, x_39, x_9, x_10, x_11, x_12, x_13, x_14, x_28); -lean_dec(x_20); -return x_40; +lean_object* x_57; lean_object* x_58; +lean_dec(x_2); +x_57 = lean_box(0); +x_58 = l_Lean_Elab_Command_accLevelAtCtor___lambda__2(x_14, x_34, x_4, x_3, x_43, x_57, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_46); +return x_58; } } else { -uint8_t x_41; -lean_dec(x_25); -lean_dec(x_20); +uint8_t x_59; +lean_dec(x_43); +lean_dec(x_34); lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); -x_41 = !lean_is_exclusive(x_26); -if (x_41 == 0) +x_59 = !lean_is_exclusive(x_44); +if (x_59 == 0) { -return x_26; +return x_44; } else { -lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_ctor_get(x_26, 0); -x_43 = lean_ctor_get(x_26, 1); -lean_inc(x_43); -lean_inc(x_42); -lean_dec(x_26); -x_44 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_44, 0, x_42); -lean_ctor_set(x_44, 1, x_43); -return x_44; +lean_object* x_60; lean_object* x_61; lean_object* x_62; +x_60 = lean_ctor_get(x_44, 0); +x_61 = lean_ctor_get(x_44, 1); +lean_inc(x_61); +lean_inc(x_60); +lean_dec(x_44); +x_62 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_62, 0, x_60); +lean_ctor_set(x_62, 1, x_61); +return x_62; } } } else { -lean_object* x_45; lean_object* x_46; +uint8_t x_63; +lean_free_object(x_27); +lean_free_object(x_23); +lean_free_object(x_19); lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_45 = lean_box(0); -x_46 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_46, 0, x_45); -lean_ctor_set(x_46, 1, x_15); -return x_46; +lean_dec(x_1); +x_63 = !lean_is_exclusive(x_33); +if (x_63 == 0) +{ +return x_33; } +else +{ +lean_object* x_64; lean_object* x_65; lean_object* x_66; +x_64 = lean_ctor_get(x_33, 0); +x_65 = lean_ctor_get(x_33, 1); +lean_inc(x_65); +lean_inc(x_64); +lean_dec(x_33); +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; } } -case 5: -{ -switch (lean_obj_tag(x_8)) { -case 0: +} +else { -lean_object* x_47; lean_object* x_48; -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_47 = lean_ctor_get(x_7, 0); -lean_inc(x_47); -lean_dec(x_7); -x_48 = l_Lean_assignLevelMVar___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___spec__1(x_47, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +uint8_t x_67; +lean_free_object(x_27); +lean_dec(x_29); +lean_free_object(x_23); +lean_free_object(x_19); lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -return x_48; -} -case 4: -{ -lean_object* x_49; lean_object* x_50; +lean_dec(x_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_49 = lean_ctor_get(x_7, 0); -lean_inc(x_49); -lean_dec(x_7); -x_50 = l_Lean_assignLevelMVar___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___spec__1(x_49, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -return x_50; -} -default: -{ -uint8_t x_51; -lean_dec(x_8); -lean_dec(x_7); -x_51 = l_Lean_Level_geq(x_2, x_6); -if (x_51 == 0) -{ -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; -x_52 = lean_ctor_get(x_3, 0); -lean_inc(x_52); -lean_dec(x_3); -lean_inc(x_52); -x_53 = l_Lean_MessageData_ofName(x_52); -x_54 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___closed__2; -x_55 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_55, 0, x_54); -lean_ctor_set(x_55, 1, x_53); -x_56 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___closed__4; -x_57 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_57, 0, x_55); -lean_ctor_set(x_57, 1, x_56); -lean_inc(x_11); -x_58 = l_Lean_Meta_getFVarLocalDecl(x_4, x_11, x_12, x_13, x_14, x_15); -if (lean_obj_tag(x_58) == 0) -{ -lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; -x_59 = lean_ctor_get(x_58, 0); -lean_inc(x_59); -x_60 = lean_ctor_get(x_58, 1); -lean_inc(x_60); -lean_dec(x_58); -x_61 = l_Lean_LocalDecl_userName(x_59); -lean_dec(x_59); -x_62 = l_Lean_Name_hasMacroScopes(x_61); -lean_dec(x_61); -if (x_62 == 0) +lean_dec(x_1); +x_67 = !lean_is_exclusive(x_31); +if (x_67 == 0) { -lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; -x_63 = l_Lean_MessageData_ofExpr(x_4); -x_64 = l_Lean_Elab_Command_accLevelAtCtor___closed__8; -x_65 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_65, 0, x_64); -lean_ctor_set(x_65, 1, x_63); -x_66 = l_Lean_Elab_Command_accLevelAtCtor___closed__10; -x_67 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_67, 0, x_65); -lean_ctor_set(x_67, 1, x_66); -x_68 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_68, 0, x_57); -lean_ctor_set(x_68, 1, x_67); +lean_object* x_68; lean_object* x_69; +x_68 = lean_ctor_get(x_31, 0); +lean_dec(x_68); x_69 = lean_box(0); -x_70 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1(x_5, x_6, x_2, x_1, x_52, x_68, x_69, x_9, x_10, x_11, x_12, x_13, x_14, x_60); -lean_dec(x_52); -return x_70; +lean_ctor_set(x_31, 0, x_69); +return x_31; } else { -lean_object* x_71; lean_object* x_72; -lean_dec(x_4); +lean_object* x_70; lean_object* x_71; lean_object* x_72; +x_70 = lean_ctor_get(x_31, 1); +lean_inc(x_70); +lean_dec(x_31); x_71 = lean_box(0); -x_72 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1(x_5, x_6, x_2, x_1, x_52, x_57, x_71, x_9, x_10, x_11, x_12, x_13, x_14, x_60); -lean_dec(x_52); +x_72 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_72, 0, x_71); +lean_ctor_set(x_72, 1, x_70); return x_72; } } +} else { -uint8_t x_73; -lean_dec(x_57); -lean_dec(x_52); -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_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); -x_73 = !lean_is_exclusive(x_58); -if (x_73 == 0) -{ -return x_58; -} -else -{ -lean_object* x_74; lean_object* x_75; lean_object* x_76; -x_74 = lean_ctor_get(x_58, 0); -x_75 = lean_ctor_get(x_58, 1); -lean_inc(x_75); +lean_object* x_73; lean_object* x_74; lean_object* x_75; +x_73 = lean_ctor_get(x_27, 0); +x_74 = lean_ctor_get(x_27, 1); lean_inc(x_74); -lean_dec(x_58); -x_76 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_76, 0, x_74); -lean_ctor_set(x_76, 1, x_75); -return x_76; -} -} -} -else -{ -lean_object* x_77; lean_object* x_78; -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_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_77 = lean_box(0); -x_78 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_78, 0, x_77); -lean_ctor_set(x_78, 1, x_15); -return x_78; -} -} -} -} -default: +lean_inc(x_73); +lean_dec(x_27); +x_75 = lean_st_ref_set(x_5, x_74, x_26); +if (lean_obj_tag(x_73) == 0) { -uint8_t x_79; -lean_dec(x_8); -lean_dec(x_7); -x_79 = l_Lean_Level_geq(x_2, x_6); -if (x_79 == 0) +lean_object* x_76; lean_object* x_77; +x_76 = lean_ctor_get(x_75, 1); +lean_inc(x_76); +lean_dec(x_75); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_14); +x_77 = lean_infer_type(x_14, x_8, x_9, x_10, x_11, x_76); +if (lean_obj_tag(x_77) == 0) { -lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; -x_80 = lean_ctor_get(x_3, 0); -lean_inc(x_80); -lean_dec(x_3); +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_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_ctor_get(x_1, 0); lean_inc(x_80); x_81 = l_Lean_MessageData_ofName(x_80); -x_82 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___closed__2; +x_82 = l_Lean_Elab_Command_accLevelAtCtor___closed__2; x_83 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_83, 0, x_82); lean_ctor_set(x_83, 1, x_81); -x_84 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___closed__4; -x_85 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_85, 0, x_83); -lean_ctor_set(x_85, 1, x_84); -lean_inc(x_11); -x_86 = l_Lean_Meta_getFVarLocalDecl(x_4, x_11, x_12, x_13, x_14, x_15); -if (lean_obj_tag(x_86) == 0) +x_84 = l_Lean_Elab_Command_accLevelAtCtor___closed__4; +lean_ctor_set_tag(x_23, 7); +lean_ctor_set(x_23, 1, x_84); +lean_ctor_set(x_23, 0, x_83); +x_85 = lean_ctor_get(x_1, 1); +lean_inc(x_85); +lean_dec(x_1); +x_86 = l_Lean_indentExpr(x_85); +lean_ctor_set_tag(x_19, 7); +lean_ctor_set(x_19, 1, x_86); +lean_ctor_set(x_19, 0, x_23); +x_87 = l_Lean_Elab_Command_accLevelAtCtor___closed__6; +x_88 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_88, 0, x_19); +lean_ctor_set(x_88, 1, x_87); +lean_inc(x_8); +x_89 = l_Lean_Meta_getFVarLocalDecl(x_2, x_8, x_9, x_10, x_11, x_79); +if (lean_obj_tag(x_89) == 0) { -lean_object* x_87; lean_object* x_88; lean_object* x_89; uint8_t 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 = l_Lean_LocalDecl_userName(x_87); -lean_dec(x_87); -x_90 = l_Lean_Name_hasMacroScopes(x_89); +lean_object* x_90; lean_object* x_91; lean_object* x_92; uint8_t x_93; +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); -if (x_90 == 0) +x_92 = l_Lean_LocalDecl_userName(x_90); +lean_dec(x_90); +x_93 = l_Lean_Name_hasMacroScopes(x_92); +lean_dec(x_92); +if (x_93 == 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; -x_91 = l_Lean_MessageData_ofExpr(x_4); -x_92 = l_Lean_Elab_Command_accLevelAtCtor___closed__8; -x_93 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_93, 0, x_92); -lean_ctor_set(x_93, 1, x_91); -x_94 = l_Lean_Elab_Command_accLevelAtCtor___closed__10; -x_95 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_95, 0, x_93); -lean_ctor_set(x_95, 1, x_94); +lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; +x_94 = l_Lean_MessageData_ofExpr(x_2); +x_95 = l_Lean_Elab_Command_accLevelAtCtor___closed__8; x_96 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_96, 0, x_85); -lean_ctor_set(x_96, 1, x_95); -x_97 = lean_box(0); -x_98 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1(x_5, x_6, x_2, x_1, x_80, x_96, x_97, x_9, x_10, x_11, x_12, x_13, x_14, x_88); -lean_dec(x_80); -return x_98; +lean_ctor_set(x_96, 0, x_95); +lean_ctor_set(x_96, 1, x_94); +x_97 = l_Lean_Elab_Command_accLevelAtCtor___closed__10; +x_98 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_98, 0, x_96); +lean_ctor_set(x_98, 1, x_97); +x_99 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_99, 0, x_88); +lean_ctor_set(x_99, 1, x_98); +x_100 = lean_box(0); +x_101 = l_Lean_Elab_Command_accLevelAtCtor___lambda__2(x_14, x_78, x_4, x_3, x_99, x_100, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_91); +return x_101; } else { -lean_object* x_99; lean_object* x_100; -lean_dec(x_4); -x_99 = lean_box(0); -x_100 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1(x_5, x_6, x_2, x_1, x_80, x_85, x_99, x_9, x_10, x_11, x_12, x_13, x_14, x_88); -lean_dec(x_80); -return x_100; +lean_object* x_102; lean_object* x_103; +lean_dec(x_2); +x_102 = lean_box(0); +x_103 = l_Lean_Elab_Command_accLevelAtCtor___lambda__2(x_14, x_78, x_4, x_3, x_88, x_102, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_91); +return x_103; } } else { -uint8_t x_101; -lean_dec(x_85); -lean_dec(x_80); +lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; +lean_dec(x_88); +lean_dec(x_78); lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); -x_101 = !lean_is_exclusive(x_86); -if (x_101 == 0) -{ -return x_86; +x_104 = lean_ctor_get(x_89, 0); +lean_inc(x_104); +x_105 = lean_ctor_get(x_89, 1); +lean_inc(x_105); +if (lean_is_exclusive(x_89)) { + lean_ctor_release(x_89, 0); + lean_ctor_release(x_89, 1); + x_106 = x_89; +} else { + lean_dec_ref(x_89); + x_106 = lean_box(0); } -else -{ -lean_object* x_102; lean_object* x_103; lean_object* x_104; -x_102 = lean_ctor_get(x_86, 0); -x_103 = lean_ctor_get(x_86, 1); -lean_inc(x_103); -lean_inc(x_102); -lean_dec(x_86); -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; +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; } } else { -lean_object* x_105; lean_object* x_106; +lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; +lean_free_object(x_23); +lean_free_object(x_19); lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_105 = lean_box(0); -x_106 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_106, 0, x_105); -lean_ctor_set(x_106, 1, x_15); -return x_106; -} +lean_dec(x_1); +x_108 = lean_ctor_get(x_77, 0); +lean_inc(x_108); +x_109 = lean_ctor_get(x_77, 1); +lean_inc(x_109); +if (lean_is_exclusive(x_77)) { + lean_ctor_release(x_77, 0); + lean_ctor_release(x_77, 1); + x_110 = x_77; +} else { + lean_dec_ref(x_77); + x_110 = lean_box(0); } +if (lean_is_scalar(x_110)) { + x_111 = lean_alloc_ctor(1, 2, 0); +} else { + x_111 = x_110; } +lean_ctor_set(x_111, 0, x_108); +lean_ctor_set(x_111, 1, x_109); +return x_111; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { -_start: +else { -size_t x_15; size_t x_16; lean_object* x_17; -x_15 = lean_unbox_usize(x_5); -lean_dec(x_5); -x_16 = lean_unbox_usize(x_6); +lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; +lean_dec(x_73); +lean_free_object(x_23); +lean_free_object(x_19); +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); -x_17 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___spec__2(x_1, x_2, x_3, x_4, x_15, x_16, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_5); lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); lean_dec(x_1); -return x_17; +x_112 = lean_ctor_get(x_75, 1); +lean_inc(x_112); +if (lean_is_exclusive(x_75)) { + lean_ctor_release(x_75, 0); + lean_ctor_release(x_75, 1); + x_113 = x_75; +} else { + lean_dec_ref(x_75); + x_113 = lean_box(0); +} +x_114 = lean_box(0); +if (lean_is_scalar(x_113)) { + x_115 = lean_alloc_ctor(0, 2, 0); +} else { + x_115 = x_113; } +lean_ctor_set(x_115, 0, x_114); +lean_ctor_set(x_115, 1, x_112); +return x_115; } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___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) { -_start: -{ -size_t x_15; size_t x_16; lean_object* x_17; -x_15 = lean_unbox_usize(x_5); -lean_dec(x_5); -x_16 = lean_unbox_usize(x_6); -lean_dec(x_6); -x_17 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___spec__3(x_1, x_2, x_3, x_4, x_15, x_16, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -lean_dec(x_4); -lean_dec(x_1); -return x_17; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_withCtorRef___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +else { -lean_object* x_10; -x_10 = l_Lean_Elab_Command_withCtorRef___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_2); -return x_10; +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 = lean_ctor_get(x_23, 0); +x_117 = lean_ctor_get(x_23, 1); +lean_inc(x_117); +lean_inc(x_116); +lean_dec(x_23); +lean_inc(x_4); +x_118 = l_Lean_Elab_Command_accLevel_go(x_3, x_21, x_4, x_116); +x_119 = lean_ctor_get(x_118, 0); +lean_inc(x_119); +x_120 = lean_ctor_get(x_118, 1); +lean_inc(x_120); +if (lean_is_exclusive(x_118)) { + lean_ctor_release(x_118, 0); + lean_ctor_release(x_118, 1); + x_121 = x_118; +} else { + lean_dec_ref(x_118); + x_121 = lean_box(0); } +x_122 = lean_st_ref_set(x_5, x_120, x_117); +if (lean_obj_tag(x_119) == 0) +{ +lean_object* x_123; lean_object* x_124; +x_123 = lean_ctor_get(x_122, 1); +lean_inc(x_123); +lean_dec(x_122); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_14); +x_124 = lean_infer_type(x_14, x_8, x_9, x_10, x_11, x_123); +if (lean_obj_tag(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; lean_object* x_137; +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 = lean_ctor_get(x_1, 0); +lean_inc(x_127); +x_128 = l_Lean_MessageData_ofName(x_127); +x_129 = l_Lean_Elab_Command_accLevelAtCtor___closed__2; +if (lean_is_scalar(x_121)) { + x_130 = lean_alloc_ctor(7, 2, 0); +} else { + x_130 = x_121; + lean_ctor_set_tag(x_130, 7); } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_withCtorRef___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___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_ctor_set(x_130, 0, x_129); +lean_ctor_set(x_130, 1, x_128); +x_131 = l_Lean_Elab_Command_accLevelAtCtor___closed__4; +x_132 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_132, 0, x_130); +lean_ctor_set(x_132, 1, x_131); +x_133 = lean_ctor_get(x_1, 1); +lean_inc(x_133); +lean_dec(x_1); +x_134 = l_Lean_indentExpr(x_133); +lean_ctor_set_tag(x_19, 7); +lean_ctor_set(x_19, 1, x_134); +lean_ctor_set(x_19, 0, x_132); +x_135 = l_Lean_Elab_Command_accLevelAtCtor___closed__6; +x_136 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_136, 0, x_19); +lean_ctor_set(x_136, 1, x_135); +lean_inc(x_8); +x_137 = l_Lean_Meta_getFVarLocalDecl(x_2, x_8, x_9, x_10, x_11, x_126); +if (lean_obj_tag(x_137) == 0) { -lean_object* x_11; -x_11 = l_Lean_Elab_Command_withCtorRef___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_object* x_138; lean_object* x_139; lean_object* x_140; uint8_t x_141; +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_LocalDecl_userName(x_138); +lean_dec(x_138); +x_141 = l_Lean_Name_hasMacroScopes(x_140); +lean_dec(x_140); +if (x_141 == 0) +{ +lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; +x_142 = l_Lean_MessageData_ofExpr(x_2); +x_143 = l_Lean_Elab_Command_accLevelAtCtor___closed__8; +x_144 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_144, 0, x_143); +lean_ctor_set(x_144, 1, x_142); +x_145 = l_Lean_Elab_Command_accLevelAtCtor___closed__10; +x_146 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_146, 0, x_144); +lean_ctor_set(x_146, 1, x_145); +x_147 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_147, 0, x_136); +lean_ctor_set(x_147, 1, x_146); +x_148 = lean_box(0); +x_149 = l_Lean_Elab_Command_accLevelAtCtor___lambda__2(x_14, x_125, x_4, x_3, x_147, x_148, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_139); +return x_149; +} +else +{ +lean_object* x_150; lean_object* x_151; lean_dec(x_2); -lean_dec(x_1); -return x_11; +x_150 = lean_box(0); +x_151 = l_Lean_Elab_Command_accLevelAtCtor___lambda__2(x_14, x_125, x_4, x_3, x_136, x_150, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_139); +return x_151; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { -_start: +else { -lean_object* x_15; -x_15 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___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_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; +lean_dec(x_136); +lean_dec(x_125); +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); -return x_15; +lean_dec(x_3); +lean_dec(x_2); +x_152 = lean_ctor_get(x_137, 0); +lean_inc(x_152); +x_153 = lean_ctor_get(x_137, 1); +lean_inc(x_153); +if (lean_is_exclusive(x_137)) { + lean_ctor_release(x_137, 0); + lean_ctor_release(x_137, 1); + x_154 = x_137; +} else { + lean_dec_ref(x_137); + x_154 = lean_box(0); } +if (lean_is_scalar(x_154)) { + x_155 = lean_alloc_ctor(1, 2, 0); +} else { + x_155 = x_154; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { -_start: -{ -lean_object* x_16; -x_16 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check(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_1); -return x_16; +lean_ctor_set(x_155, 0, x_152); +lean_ctor_set(x_155, 1, x_153); +return x_155; } } -LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { -_start: -{ -uint8_t x_15; -x_15 = lean_usize_dec_lt(x_6, x_5); -if (x_15 == 0) +else { -lean_object* x_16; -lean_dec(x_13); -lean_dec(x_12); +lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; +lean_dec(x_121); +lean_free_object(x_19); +lean_dec(x_14); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_16 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_16, 0, x_7); -lean_ctor_set(x_16, 1, x_14); -return x_16; +lean_dec(x_1); +x_156 = lean_ctor_get(x_124, 0); +lean_inc(x_156); +x_157 = lean_ctor_get(x_124, 1); +lean_inc(x_157); +if (lean_is_exclusive(x_124)) { + lean_ctor_release(x_124, 0); + lean_ctor_release(x_124, 1); + x_158 = x_124; +} else { + lean_dec_ref(x_124); + x_158 = lean_box(0); +} +if (lean_is_scalar(x_158)) { + x_159 = lean_alloc_ctor(1, 2, 0); +} else { + x_159 = x_158; +} +lean_ctor_set(x_159, 0, x_156); +lean_ctor_set(x_159, 1, x_157); +return x_159; +} } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; +lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; +lean_dec(x_121); +lean_dec(x_119); +lean_free_object(x_19); +lean_dec(x_14); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); lean_dec(x_7); -x_17 = lean_ctor_get(x_4, 0); -x_18 = lean_array_uget(x_17, x_6); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_18); -x_19 = lean_infer_type(x_18, x_10, x_11, x_12, x_13, x_14); -if (lean_obj_tag(x_19) == 0) +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_160 = lean_ctor_get(x_122, 1); +lean_inc(x_160); +if (lean_is_exclusive(x_122)) { + lean_ctor_release(x_122, 0); + lean_ctor_release(x_122, 1); + x_161 = x_122; +} else { + lean_dec_ref(x_122); + x_161 = lean_box(0); +} +x_162 = lean_box(0); +if (lean_is_scalar(x_161)) { + x_163 = lean_alloc_ctor(0, 2, 0); +} else { + x_163 = x_161; +} +lean_ctor_set(x_163, 0, x_162); +lean_ctor_set(x_163, 1, x_160); +return x_163; +} +} +} +else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_19, 1); -lean_inc(x_21); +lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; +x_164 = lean_ctor_get(x_19, 0); +x_165 = lean_ctor_get(x_19, 1); +lean_inc(x_165); +lean_inc(x_164); lean_dec(x_19); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_20); -x_22 = l_Lean_Meta_getLevel(x_20, x_10, x_11, x_12, x_13, x_21); -if (lean_obj_tag(x_22) == 0) +x_166 = lean_st_ref_take(x_5, x_165); +x_167 = lean_ctor_get(x_166, 0); +lean_inc(x_167); +x_168 = lean_ctor_get(x_166, 1); +lean_inc(x_168); +if (lean_is_exclusive(x_166)) { + lean_ctor_release(x_166, 0); + lean_ctor_release(x_166, 1); + x_169 = x_166; +} else { + lean_dec_ref(x_166); + x_169 = lean_box(0); +} +lean_inc(x_4); +x_170 = l_Lean_Elab_Command_accLevel_go(x_3, x_164, x_4, x_167); +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; +} else { + lean_dec_ref(x_170); + x_173 = lean_box(0); +} +x_174 = lean_st_ref_set(x_5, x_172, x_168); +if (lean_obj_tag(x_171) == 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; -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_instantiateLevelMVars___at_Lean_Elab_Command_shouldInferResultUniverse___spec__1(x_23, x_8, x_9, x_10, x_11, x_12, x_13, x_24); -x_26 = lean_ctor_get(x_25, 0); -lean_inc(x_26); -x_27 = lean_ctor_get(x_25, 1); -lean_inc(x_27); -lean_dec(x_25); -x_28 = l_Lean_Level_normalize(x_26); -lean_dec(x_26); -lean_inc(x_13); -lean_inc(x_12); +lean_object* x_175; lean_object* x_176; +x_175 = lean_ctor_get(x_174, 1); +lean_inc(x_175); +lean_dec(x_174); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -lean_inc(x_28); -lean_inc(x_3); -lean_inc_n(x_2, 2); -x_29 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check(x_1, x_2, x_3, x_18, x_20, x_28, x_28, x_2, x_8, x_9, x_10, x_11, x_12, x_13, x_27); -if (lean_obj_tag(x_29) == 0) +lean_inc(x_14); +x_176 = lean_infer_type(x_14, x_8, x_9, x_10, x_11, x_175); +if (lean_obj_tag(x_176) == 0) { -lean_object* x_30; size_t x_31; size_t x_32; lean_object* x_33; -x_30 = lean_ctor_get(x_29, 1); -lean_inc(x_30); -lean_dec(x_29); -x_31 = 1; -x_32 = lean_usize_add(x_6, x_31); -x_33 = lean_box(0); -x_6 = x_32; -x_7 = x_33; -x_14 = x_30; -goto _start; +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; +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_ctor_get(x_1, 0); +lean_inc(x_179); +x_180 = l_Lean_MessageData_ofName(x_179); +x_181 = l_Lean_Elab_Command_accLevelAtCtor___closed__2; +if (lean_is_scalar(x_173)) { + x_182 = lean_alloc_ctor(7, 2, 0); +} else { + x_182 = x_173; + lean_ctor_set_tag(x_182, 7); } -else +lean_ctor_set(x_182, 0, x_181); +lean_ctor_set(x_182, 1, x_180); +x_183 = l_Lean_Elab_Command_accLevelAtCtor___closed__4; +if (lean_is_scalar(x_169)) { + x_184 = lean_alloc_ctor(7, 2, 0); +} else { + x_184 = x_169; + lean_ctor_set_tag(x_184, 7); +} +lean_ctor_set(x_184, 0, x_182); +lean_ctor_set(x_184, 1, x_183); +x_185 = lean_ctor_get(x_1, 1); +lean_inc(x_185); +lean_dec(x_1); +x_186 = l_Lean_indentExpr(x_185); +x_187 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_187, 0, x_184); +lean_ctor_set(x_187, 1, x_186); +x_188 = l_Lean_Elab_Command_accLevelAtCtor___closed__6; +x_189 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_189, 0, x_187); +lean_ctor_set(x_189, 1, x_188); +lean_inc(x_8); +x_190 = l_Lean_Meta_getFVarLocalDecl(x_2, x_8, x_9, x_10, x_11, x_178); +if (lean_obj_tag(x_190) == 0) { -uint8_t x_35; -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_3); -lean_dec(x_2); -x_35 = !lean_is_exclusive(x_29); -if (x_35 == 0) +lean_object* x_191; lean_object* x_192; lean_object* x_193; uint8_t x_194; +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_LocalDecl_userName(x_191); +lean_dec(x_191); +x_194 = l_Lean_Name_hasMacroScopes(x_193); +lean_dec(x_193); +if (x_194 == 0) { -return x_29; +lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; +x_195 = l_Lean_MessageData_ofExpr(x_2); +x_196 = l_Lean_Elab_Command_accLevelAtCtor___closed__8; +x_197 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_197, 0, x_196); +lean_ctor_set(x_197, 1, x_195); +x_198 = l_Lean_Elab_Command_accLevelAtCtor___closed__10; +x_199 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_199, 0, x_197); +lean_ctor_set(x_199, 1, x_198); +x_200 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_200, 0, x_189); +lean_ctor_set(x_200, 1, x_199); +x_201 = lean_box(0); +x_202 = l_Lean_Elab_Command_accLevelAtCtor___lambda__2(x_14, x_177, x_4, x_3, x_200, x_201, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_192); +return x_202; } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_29, 0); -x_37 = lean_ctor_get(x_29, 1); -lean_inc(x_37); -lean_inc(x_36); -lean_dec(x_29); -x_38 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -return x_38; -} +lean_object* x_203; lean_object* x_204; +lean_dec(x_2); +x_203 = lean_box(0); +x_204 = l_Lean_Elab_Command_accLevelAtCtor___lambda__2(x_14, x_177, x_4, x_3, x_189, x_203, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_192); +return x_204; } } else { -uint8_t x_39; -lean_dec(x_20); -lean_dec(x_18); -lean_dec(x_13); -lean_dec(x_12); +lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; +lean_dec(x_189); +lean_dec(x_177); +lean_dec(x_14); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_39 = !lean_is_exclusive(x_22); -if (x_39 == 0) -{ -return x_22; +x_205 = lean_ctor_get(x_190, 0); +lean_inc(x_205); +x_206 = lean_ctor_get(x_190, 1); +lean_inc(x_206); +if (lean_is_exclusive(x_190)) { + lean_ctor_release(x_190, 0); + lean_ctor_release(x_190, 1); + x_207 = x_190; +} else { + lean_dec_ref(x_190); + x_207 = lean_box(0); } -else -{ -lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_40 = lean_ctor_get(x_22, 0); -x_41 = lean_ctor_get(x_22, 1); -lean_inc(x_41); -lean_inc(x_40); -lean_dec(x_22); -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; +if (lean_is_scalar(x_207)) { + x_208 = lean_alloc_ctor(1, 2, 0); +} else { + x_208 = x_207; } +lean_ctor_set(x_208, 0, x_205); +lean_ctor_set(x_208, 1, x_206); +return x_208; } } else { -uint8_t x_43; -lean_dec(x_18); -lean_dec(x_13); -lean_dec(x_12); +lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; +lean_dec(x_173); +lean_dec(x_169); +lean_dec(x_14); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_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; -} -} -} -} -} -LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses___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; lean_object* x_16; size_t x_17; lean_object* x_18; size_t x_19; lean_object* x_20; lean_object* x_21; -x_14 = lean_array_get_size(x_5); -x_15 = l_Array_toSubarray___rarg(x_5, x_1, x_14); -x_16 = lean_ctor_get(x_15, 2); -lean_inc(x_16); -x_17 = lean_usize_of_nat(x_16); -lean_dec(x_16); -x_18 = lean_ctor_get(x_15, 1); -lean_inc(x_18); -x_19 = lean_usize_of_nat(x_18); -lean_dec(x_18); -x_20 = lean_box(0); -x_21 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses___spec__1(x_2, x_3, x_4, x_15, x_17, x_19, x_20, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_15); -if (lean_obj_tag(x_21) == 0) -{ -uint8_t x_22; -x_22 = !lean_is_exclusive(x_21); -if (x_22 == 0) -{ -lean_object* x_23; -x_23 = lean_ctor_get(x_21, 0); -lean_dec(x_23); -lean_ctor_set(x_21, 0, x_20); -return x_21; +lean_dec(x_1); +x_209 = lean_ctor_get(x_176, 0); +lean_inc(x_209); +x_210 = lean_ctor_get(x_176, 1); +lean_inc(x_210); +if (lean_is_exclusive(x_176)) { + lean_ctor_release(x_176, 0); + lean_ctor_release(x_176, 1); + x_211 = x_176; +} else { + lean_dec_ref(x_176); + x_211 = lean_box(0); } -else -{ -lean_object* x_24; lean_object* x_25; -x_24 = lean_ctor_get(x_21, 1); -lean_inc(x_24); -lean_dec(x_21); -x_25 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_25, 0, x_20); -lean_ctor_set(x_25, 1, x_24); -return x_25; +if (lean_is_scalar(x_211)) { + x_212 = lean_alloc_ctor(1, 2, 0); +} else { + x_212 = x_211; } +lean_ctor_set(x_212, 0, x_209); +lean_ctor_set(x_212, 1, x_210); +return x_212; } -else -{ -uint8_t x_26; -x_26 = !lean_is_exclusive(x_21); -if (x_26 == 0) -{ -return x_21; } else { -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_21, 0); -x_28 = lean_ctor_get(x_21, 1); -lean_inc(x_28); -lean_inc(x_27); -lean_dec(x_21); -x_29 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_29, 0, x_27); -lean_ctor_set(x_29, 1, x_28); -return x_29; -} -} -} -} -LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -if (lean_obj_tag(x_4) == 0) -{ -lean_object* x_12; lean_object* x_13; +lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; +lean_dec(x_173); +lean_dec(x_171); +lean_dec(x_169); +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_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; +x_213 = lean_ctor_get(x_174, 1); +lean_inc(x_213); +if (lean_is_exclusive(x_174)) { + lean_ctor_release(x_174, 0); + lean_ctor_release(x_174, 1); + x_214 = x_174; +} else { + lean_dec_ref(x_174); + x_214 = lean_box(0); +} +x_215 = lean_box(0); +if (lean_is_scalar(x_214)) { + x_216 = lean_alloc_ctor(0, 2, 0); +} else { + x_216 = x_214; +} +lean_ctor_set(x_216, 0, x_215); +lean_ctor_set(x_216, 1, x_213); +return x_216; +} } -else -{ -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_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); -x_16 = lean_ctor_get(x_14, 1); -lean_inc(x_16); -lean_inc(x_3); -lean_inc(x_1); -lean_inc(x_2); -x_17 = lean_alloc_closure((void*)(l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses___spec__2___lambda__1___boxed), 13, 4); -lean_closure_set(x_17, 0, x_2); -lean_closure_set(x_17, 1, x_1); -lean_closure_set(x_17, 2, x_3); -lean_closure_set(x_17, 3, x_14); -x_18 = 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_19 = l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___spec__1___rarg(x_16, x_17, x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_19) == 0) -{ -lean_object* x_20; -x_20 = lean_ctor_get(x_19, 1); -lean_inc(x_20); -lean_dec(x_19); -x_4 = x_15; -x_11 = x_20; -goto _start; } else { -uint8_t x_22; -lean_dec(x_15); +uint8_t x_217; +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_22 = !lean_is_exclusive(x_19); -if (x_22 == 0) +x_217 = !lean_is_exclusive(x_16); +if (x_217 == 0) { -return x_19; +return x_16; } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_19, 0); -x_24 = lean_ctor_get(x_19, 1); -lean_inc(x_24); -lean_inc(x_23); -lean_dec(x_19); -x_25 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_25, 0, x_23); -lean_ctor_set(x_25, 1, x_24); -return x_25; -} -} +lean_object* x_218; lean_object* x_219; lean_object* x_220; +x_218 = lean_ctor_get(x_16, 0); +x_219 = lean_ctor_get(x_16, 1); +lean_inc(x_219); +lean_inc(x_218); +lean_dec(x_16); +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; } } } -LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses___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: -{ -if (lean_obj_tag(x_4) == 0) +else { -lean_object* x_12; lean_object* x_13; +uint8_t x_221; +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_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); +x_221 = !lean_is_exclusive(x_13); +if (x_221 == 0) +{ 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_4, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_4, 1); -lean_inc(x_15); -lean_dec(x_4); -x_16 = lean_ctor_get(x_14, 2); -lean_inc(x_16); -lean_dec(x_14); -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); -lean_inc(x_1); -x_17 = l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses___spec__2(x_1, x_2, x_3, x_16, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_17) == 0) -{ -lean_object* x_18; -x_18 = lean_ctor_get(x_17, 1); -lean_inc(x_18); -lean_dec(x_17); -x_4 = x_15; -x_11 = x_18; -goto _start; -} -else -{ -uint8_t x_20; -lean_dec(x_15); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_20 = !lean_is_exclusive(x_17); -if (x_20 == 0) -{ -return x_17; -} -else -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_17, 0); -x_22 = lean_ctor_get(x_17, 1); -lean_inc(x_22); -lean_inc(x_21); -lean_dec(x_17); -x_23 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_23, 0, x_21); -lean_ctor_set(x_23, 1, x_22); -return x_23; -} +lean_object* x_222; lean_object* x_223; lean_object* x_224; +x_222 = lean_ctor_get(x_13, 0); +x_223 = lean_ctor_get(x_13, 1); +lean_inc(x_223); +lean_inc(x_222); +lean_dec(x_13); +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_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_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_instantiateLevelMVars___at_Lean_Elab_Command_accLevelAtCtor___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_11; -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_11) == 0) -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; -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_instantiateLevelMVars___at_Lean_Elab_Command_shouldInferResultUniverse___spec__1(x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_13); -x_15 = lean_ctor_get(x_14, 0); -lean_inc(x_15); -x_16 = lean_ctor_get(x_14, 1); -lean_inc(x_16); -lean_dec(x_14); -x_17 = l_Lean_Level_normalize(x_15); -lean_dec(x_15); -lean_inc(x_4); -lean_inc(x_17); -x_18 = l_Lean_Elab_Command_checkResultingUniverse(x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_16); -if (lean_obj_tag(x_18) == 0) -{ -uint8_t x_19; -x_19 = !lean_is_exclusive(x_18); -if (x_19 == 0) -{ -lean_object* x_20; lean_object* x_21; uint8_t x_22; -x_20 = lean_ctor_get(x_18, 1); -x_21 = lean_ctor_get(x_18, 0); -lean_dec(x_21); -x_22 = l_Lean_Level_isZero(x_17); -if (x_22 == 0) -{ -lean_object* x_23; -lean_free_object(x_18); -x_23 = l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses___spec__3(x_1, x_2, x_17, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_20); -return x_23; -} -else -{ -lean_object* x_24; -lean_dec(x_17); -lean_dec(x_9); +lean_object* x_10; +x_10 = l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_accLevelAtCtor___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -18451,30 +19236,14 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_24 = lean_box(0); -lean_ctor_set(x_18, 0, x_24); -return x_18; -} +return x_10; } -else -{ -lean_object* x_25; uint8_t x_26; -x_25 = lean_ctor_get(x_18, 1); -lean_inc(x_25); -lean_dec(x_18); -x_26 = l_Lean_Level_isZero(x_17); -if (x_26 == 0) -{ -lean_object* x_27; -x_27 = l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses___spec__3(x_1, x_2, x_17, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_25); -return x_27; } -else +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_accLevelAtCtor___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: { -lean_object* x_28; lean_object* x_29; -lean_dec(x_17); -lean_dec(x_9); +lean_object* x_10; +x_10 = l_Lean_throwError___at_Lean_Elab_Command_accLevelAtCtor___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -18482,19 +19251,14 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -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_25); -return x_29; -} +return x_10; } } -else +LEAN_EXPORT lean_object* l_Lean_Elab_Command_accLevelAtCtor___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_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_30; -lean_dec(x_17); +lean_object* x_11; +x_11 = l_Lean_Elab_Command_accLevelAtCtor___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); @@ -18503,5097 +19267,4843 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_30 = !lean_is_exclusive(x_18); -if (x_30 == 0) -{ -return x_18; +return x_11; } -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_Lean_Elab_Command_accLevelAtCtor___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; +x_15 = l_Lean_Elab_Command_accLevelAtCtor___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; } } -else +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___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, lean_object* x_7, lean_object* x_8, size_t x_9, lean_object* x_10) { +_start: { -uint8_t x_34; -lean_dec(x_9); +if (lean_obj_tag(x_10) == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_dec(x_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_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +lean_dec(x_10); +x_12 = lean_ctor_get(x_1, 0); +lean_inc(x_12); lean_dec(x_1); -x_34 = !lean_is_exclusive(x_11); -if (x_34 == 0) -{ -return x_11; +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_11); +return x_14; } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_35 = lean_ctor_get(x_11, 0); -x_36 = lean_ctor_get(x_11, 1); -lean_inc(x_36); -lean_inc(x_35); -lean_dec(x_11); -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_15; size_t x_16; size_t x_17; lean_object* x_18; +x_15 = lean_ctor_get(x_10, 0); +lean_inc(x_15); +lean_dec(x_10); +x_16 = 1; +x_17 = lean_usize_add(x_2, x_16); +x_18 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_17, x_15); +return x_18; } } } -LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -size_t x_15; size_t x_16; lean_object* x_17; -x_15 = lean_unbox_usize(x_5); -lean_dec(x_5); -x_16 = lean_unbox_usize(x_6); -lean_dec(x_6); -x_17 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses___spec__1(x_1, x_2, x_3, x_4, x_15, x_16, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -lean_dec(x_4); -lean_dec(x_1); -return x_17; +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_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses___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) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___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_14; -x_14 = l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses___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_6); +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); -return x_14; +x_7 = lean_apply_3(x_6, lean_box(0), x_5, x_3); +return x_7; } } -LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUsed___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg___lambda__4(lean_object* x_1, lean_object* x_2) { _start: { -if (lean_obj_tag(x_1) == 0) -{ -lean_object* x_8; lean_object* x_9; -x_8 = lean_box(0); -x_9 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_9, 0, x_8); -lean_ctor_set(x_9, 1, x_7); -return x_9; -} -else -{ -lean_object* 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); -x_11 = lean_ctor_get(x_1, 1); -lean_inc(x_11); +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_3 = lean_ctor_get(x_1, 0); +lean_inc(x_3); lean_dec(x_1); -x_12 = lean_ctor_get(x_10, 1); -lean_inc(x_12); -lean_dec(x_10); -x_13 = l_Lean_Expr_collectFVars(x_12, x_2, x_3, x_4, x_5, x_6, x_7); -x_14 = lean_ctor_get(x_13, 1); -lean_inc(x_14); -lean_dec(x_13); -x_1 = x_11; -x_7 = x_14; -goto _start; -} -} -} -LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUsed___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: -{ -if (lean_obj_tag(x_1) == 0) -{ -lean_object* x_8; lean_object* x_9; -x_8 = lean_box(0); -x_9 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_9, 0, x_8); -lean_ctor_set(x_9, 1, x_7); +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_box(0); +x_7 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_7, 0, x_5); +lean_ctor_set(x_7, 1, x_6); +x_8 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_8, 0, x_7); +x_9 = lean_apply_2(x_4, 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_1, 0); -lean_inc(x_10); -x_11 = lean_ctor_get(x_1, 1); -lean_inc(x_11); -lean_dec(x_1); -x_12 = lean_ctor_get(x_10, 1); -lean_inc(x_12); -x_13 = l_Lean_Expr_collectFVars(x_12, x_2, x_3, x_4, x_5, x_6, x_7); -x_14 = lean_ctor_get(x_13, 1); -lean_inc(x_14); -lean_dec(x_13); -x_15 = lean_ctor_get(x_10, 2); -lean_inc(x_15); -lean_dec(x_10); -x_16 = l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUsed___spec__1(x_15, x_2, x_3, x_4, x_5, x_6, x_14); -x_17 = lean_ctor_get(x_16, 1); -lean_inc(x_17); -lean_dec(x_16); -x_1 = x_11; -x_7 = x_17; -goto _start; -} } -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUsed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, size_t x_8, size_t x_9, lean_object* x_10) { _start: { -lean_object* x_8; -x_8 = l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUsed___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -return x_8; -} -} -LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUsed___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: +uint8_t x_11; +x_11 = lean_usize_dec_lt(x_9, x_8); +if (x_11 == 0) { -lean_object* x_8; -x_8 = l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUsed___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_object* 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); lean_dec(x_3); lean_dec(x_2); -return x_8; -} +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_apply_2(x_13, lean_box(0), x_10); +return x_14; } -LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUsed___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: +else { -lean_object* x_8; -x_8 = l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUsed___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -lean_dec(x_6); -lean_dec(x_5); +lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +lean_dec(x_10); +x_15 = lean_array_uget(x_7, x_9); +x_16 = lean_ctor_get(x_1, 1); +lean_inc(x_16); +x_17 = lean_ctor_get(x_15, 2); +lean_inc(x_17); +x_18 = lean_name_eq(x_17, x_3); +lean_dec(x_17); +x_19 = lean_box_usize(x_9); +x_20 = lean_box_usize(x_8); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_2); +lean_inc(x_1); +x_21 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg___lambda__1___boxed), 10, 9); +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_6); +lean_closure_set(x_21, 7, x_7); +lean_closure_set(x_21, 8, x_20); +if (x_18 == 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_15); lean_dec(x_4); -lean_dec(x_3); lean_dec(x_2); -return x_8; -} +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 = lean_box(0); +lean_inc(x_23); +x_25 = lean_apply_2(x_23, lean_box(0), x_24); +x_26 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg___lambda__2___boxed), 3, 2); +lean_closure_set(x_26, 0, x_6); +lean_closure_set(x_26, 1, x_23); +x_27 = lean_apply_4(x_5, lean_box(0), lean_box(0), x_25, x_26); +x_28 = lean_apply_4(x_16, lean_box(0), lean_box(0), x_27, x_21); +return x_28; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUsed___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: +else { -lean_object* x_8; -x_8 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUsed(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +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_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_8; +x_29 = lean_ctor_get(x_15, 0); +lean_inc(x_29); +lean_dec(x_15); +x_30 = lean_ctor_get(x_2, 0); +lean_inc(x_30); +x_31 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg___lambda__3___boxed), 4, 3); +lean_closure_set(x_31, 0, x_29); +lean_closure_set(x_31, 1, x_2); +lean_closure_set(x_31, 2, x_4); +lean_inc(x_5); +x_32 = lean_apply_4(x_5, lean_box(0), lean_box(0), x_30, x_31); +x_33 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg___lambda__4), 2, 1); +lean_closure_set(x_33, 0, x_1); +x_34 = lean_apply_4(x_5, lean_box(0), lean_box(0), x_32, x_33); +x_35 = lean_apply_4(x_16, lean_box(0), lean_box(0), x_34, x_21); +return x_35; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_removeUnused___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = lean_box(0); -x_2 = l_Lean_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__2___closed__3; -x_3 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__3___closed__1; -x_4 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_4, 0, x_2); -lean_ctor_set(x_4, 1, x_1); -lean_ctor_set(x_4, 2, x_3); -return x_4; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_removeUnused(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_10 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_removeUnused___closed__1; -x_11 = lean_st_mk_ref(x_10, 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 = l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUsed___spec__2(x_2, x_12, x_5, x_6, x_7, x_8, 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_12, x_15); -lean_dec(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_Lean_Meta_removeUnused(x_1, x_17, x_5, x_6, x_7, x_8, x_18); -return x_19; +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg___boxed), 10, 0); +return x_3; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_removeUnused___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__2___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_10; -x_10 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_removeUnused(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_object* x_5; +x_5 = lean_ctor_get(x_4, 0); +lean_inc(x_5); lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -return x_10; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withUsed___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: +if (lean_obj_tag(x_5) == 0) { -lean_object* x_11; -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_6 = lean_ctor_get(x_1, 0); lean_inc(x_6); -x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_removeUnused(x_1, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_11) == 0) -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); -x_13 = lean_ctor_get(x_12, 1); -lean_inc(x_13); -x_14 = lean_ctor_get(x_11, 1); -lean_inc(x_14); -lean_dec(x_11); -x_15 = lean_ctor_get(x_12, 0); -lean_inc(x_15); -lean_dec(x_12); -x_16 = lean_ctor_get(x_13, 0); -lean_inc(x_16); -x_17 = lean_ctor_get(x_13, 1); -lean_inc(x_17); -lean_dec(x_13); -x_18 = lean_apply_1(x_3, x_17); -x_19 = l_Lean_Meta_withLCtx___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__3___rarg(x_15, x_16, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_14); -return x_19; +lean_dec(x_1); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +x_8 = lean_box(0); +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_Command_withCtorRef___spec__1___rarg___lambda__2___boxed), 3, 2); +lean_closure_set(x_10, 0, x_2); +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; } else { -uint8_t x_20; -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); +uint8_t x_12; lean_dec(x_3); -x_20 = !lean_is_exclusive(x_11); -if (x_20 == 0) +lean_dec(x_2); +x_12 = !lean_is_exclusive(x_5); +if (x_12 == 0) { -return x_11; +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_1, 0); +lean_inc(x_13); +lean_dec(x_1); +x_14 = lean_ctor_get(x_13, 1); +lean_inc(x_14); +lean_dec(x_13); +x_15 = lean_box(0); +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_5); +lean_ctor_set(x_16, 1, x_15); +x_17 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_17, 0, x_16); +x_18 = lean_apply_2(x_14, lean_box(0), x_17); +return x_18; } 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_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_19 = lean_ctor_get(x_5, 0); +lean_inc(x_19); +lean_dec(x_5); +x_20 = lean_ctor_get(x_1, 0); +lean_inc(x_20); +lean_dec(x_1); +x_21 = lean_ctor_get(x_20, 1); 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; -} -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withUsed(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withUsed___rarg___boxed), 10, 0); -return x_2; +lean_dec(x_20); +x_22 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_22, 0, x_19); +x_23 = lean_box(0); +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); +x_25 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_25, 0, x_24); +x_26 = lean_apply_2(x_21, lean_box(0), x_25); +return x_26; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withUsed___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; -x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withUsed___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_1); -return x_11; } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateParams___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__2___rarg___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, size_t x_9, lean_object* x_10) { _start: { -if (lean_obj_tag(x_2) == 0) +if (lean_obj_tag(x_10) == 0) { -lean_object* x_11; lean_object* x_12; -lean_dec(x_9); +lean_object* x_11; lean_object* 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); +lean_dec(x_3); +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +lean_dec(x_10); +x_12 = lean_ctor_get(x_1, 0); +lean_inc(x_12); lean_dec(x_1); -x_11 = l_List_reverse___rarg(x_3); -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; +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_11); +return x_14; } else { -uint8_t x_13; -x_13 = !lean_is_exclusive(x_2); -if (x_13 == 0) -{ -lean_object* x_14; uint8_t x_15; -x_14 = lean_ctor_get(x_2, 0); -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; -x_16 = lean_ctor_get(x_2, 1); -x_17 = lean_ctor_get(x_14, 0); -x_18 = lean_ctor_get(x_14, 1); -lean_inc(x_1); -x_19 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkTypeFor___lambda__1___boxed), 9, 2); -lean_closure_set(x_19, 0, x_1); -lean_closure_set(x_19, 1, x_18); -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_20 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___rarg(x_1, x_19, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_20) == 0) -{ -lean_object* x_21; lean_object* x_22; -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_20, 1); -lean_inc(x_22); -lean_dec(x_20); -lean_ctor_set(x_14, 1, x_21); -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_22; -x_2 = _tmp_1; -x_3 = _tmp_2; -x_10 = _tmp_9; +lean_object* x_15; size_t x_16; size_t x_17; lean_object* x_18; +x_15 = lean_ctor_get(x_10, 0); +lean_inc(x_15); +lean_dec(x_10); +x_16 = 1; +x_17 = lean_usize_add(x_2, x_16); +x_18 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__2___rarg(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_17, x_15); +return x_18; } -goto _start; } -else +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, size_t x_8, size_t x_9, lean_object* x_10) { +_start: { -uint8_t x_24; -lean_free_object(x_14); -lean_dec(x_17); -lean_free_object(x_2); -lean_dec(x_16); -lean_dec(x_9); -lean_dec(x_8); +uint8_t x_11; +x_11 = lean_usize_dec_lt(x_9, x_8); +if (x_11 == 0) +{ +lean_object* 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); lean_dec(x_3); +lean_dec(x_2); +x_12 = lean_ctor_get(x_1, 0); +lean_inc(x_12); lean_dec(x_1); -x_24 = !lean_is_exclusive(x_20); -if (x_24 == 0) -{ -return x_20; +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_10); +return x_14; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_20, 0); -x_26 = lean_ctor_get(x_20, 1); -lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_20); -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_15; lean_object* x_16; lean_object* x_17; size_t x_18; size_t x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +lean_dec(x_10); +x_15 = lean_array_uget(x_7, x_9); +x_16 = lean_ctor_get(x_1, 1); +lean_inc(x_16); +x_17 = lean_ctor_get(x_15, 8); +lean_inc(x_17); +lean_dec(x_15); +x_18 = lean_array_size(x_17); +x_19 = 0; +lean_inc_n(x_6, 2); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_20 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_17, x_18, x_19, x_6); +lean_inc(x_5); +lean_inc(x_6); +lean_inc(x_1); +x_21 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__2___rarg___lambda__1), 4, 3); +lean_closure_set(x_21, 0, x_1); +lean_closure_set(x_21, 1, x_6); +lean_closure_set(x_21, 2, x_5); +lean_inc(x_5); +x_22 = lean_apply_4(x_5, lean_box(0), lean_box(0), x_20, x_21); +x_23 = lean_box_usize(x_9); +x_24 = lean_box_usize(x_8); +x_25 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__2___rarg___lambda__2___boxed), 10, 9); +lean_closure_set(x_25, 0, x_1); +lean_closure_set(x_25, 1, x_23); +lean_closure_set(x_25, 2, x_2); +lean_closure_set(x_25, 3, x_3); +lean_closure_set(x_25, 4, x_4); +lean_closure_set(x_25, 5, x_5); +lean_closure_set(x_25, 6, x_6); +lean_closure_set(x_25, 7, x_7); +lean_closure_set(x_25, 8, x_24); +x_26 = lean_apply_4(x_16, lean_box(0), lean_box(0), x_22, x_25); +return x_26; } } } -else +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__2(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__2___rarg___boxed), 10, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_withCtorRef___rarg___lambda__1(lean_object* x_1, lean_object* x_2) { +_start: { -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_2, 1); -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); lean_inc(x_1); -x_31 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkTypeFor___lambda__1___boxed), 9, 2); -lean_closure_set(x_31, 0, x_1); -lean_closure_set(x_31, 1, x_30); -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_32 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___rarg(x_1, x_31, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_32) == 0) +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_withCtorRef___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: { -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 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_35, 0, x_29); -lean_ctor_set(x_35, 1, x_33); -lean_ctor_set(x_2, 1, x_3); -lean_ctor_set(x_2, 0, x_35); +lean_object* x_5; +x_5 = lean_ctor_get(x_4, 0); +lean_inc(x_5); +lean_dec(x_4); +if (lean_obj_tag(x_5) == 0) { -lean_object* _tmp_1 = x_28; -lean_object* _tmp_2 = x_2; -lean_object* _tmp_9 = x_34; -x_2 = _tmp_1; -x_3 = _tmp_2; -x_10 = _tmp_9; -} -goto _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_alloc_closure((void*)(l_Lean_Elab_Command_withCtorRef___rarg___lambda__1___boxed), 2, 1); +lean_closure_set(x_6, 0, x_1); +x_7 = lean_ctor_get(x_2, 0); +lean_inc(x_7); +lean_dec(x_2); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_box(0); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +x_11 = lean_apply_4(x_3, lean_box(0), lean_box(0), x_10, x_6); +return x_11; } else { -lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; -lean_dec(x_29); -lean_free_object(x_2); -lean_dec(x_28); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_dec(x_3); lean_dec(x_1); -x_37 = lean_ctor_get(x_32, 0); -lean_inc(x_37); -x_38 = lean_ctor_get(x_32, 1); -lean_inc(x_38); -if (lean_is_exclusive(x_32)) { - lean_ctor_release(x_32, 0); - lean_ctor_release(x_32, 1); - x_39 = x_32; -} else { - lean_dec_ref(x_32); - x_39 = lean_box(0); +x_12 = lean_ctor_get(x_5, 0); +lean_inc(x_12); +lean_dec(x_5); +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_12); +return x_15; } -if (lean_is_scalar(x_39)) { - x_40 = lean_alloc_ctor(1, 2, 0); -} else { - x_40 = x_39; } -lean_ctor_set(x_40, 0, x_37); -lean_ctor_set(x_40, 1, x_38); -return x_40; } +static lean_object* _init_l_Lean_Elab_Command_withCtorRef___rarg___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; } } -else +LEAN_EXPORT lean_object* l_Lean_Elab_Command_withCtorRef___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_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_2, 0); -x_42 = lean_ctor_get(x_2, 1); -lean_inc(x_42); -lean_inc(x_41); -lean_dec(x_2); -x_43 = lean_ctor_get(x_41, 0); -lean_inc(x_43); -x_44 = lean_ctor_get(x_41, 1); -lean_inc(x_44); -if (lean_is_exclusive(x_41)) { - lean_ctor_release(x_41, 0); - lean_ctor_release(x_41, 1); - x_45 = x_41; -} else { - lean_dec_ref(x_41); - x_45 = lean_box(0); -} -lean_inc(x_1); -x_46 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkTypeFor___lambda__1___boxed), 9, 2); -lean_closure_set(x_46, 0, x_1); -lean_closure_set(x_46, 1, x_44); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); +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; +x_6 = lean_ctor_get(x_1, 1); +lean_inc(x_6); +x_7 = lean_array_size(x_3); +x_8 = 0; +x_9 = l_Lean_Elab_Command_withCtorRef___rarg___closed__1; lean_inc(x_6); lean_inc(x_5); -lean_inc(x_4); -x_47 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___rarg(x_1, x_46, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_47) == 0) +lean_inc(x_1); +x_10 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__2___rarg(x_1, x_2, x_4, x_5, x_6, x_9, x_3, x_7, x_8, x_9); +lean_inc(x_6); +x_11 = lean_alloc_closure((void*)(l_Lean_Elab_Command_withCtorRef___rarg___lambda__2), 4, 3); +lean_closure_set(x_11, 0, x_5); +lean_closure_set(x_11, 1, x_1); +lean_closure_set(x_11, 2, x_6); +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_Elab_Command_withCtorRef(lean_object* x_1, lean_object* x_2) { +_start: { -lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_48 = lean_ctor_get(x_47, 0); -lean_inc(x_48); -x_49 = lean_ctor_get(x_47, 1); -lean_inc(x_49); -lean_dec(x_47); -if (lean_is_scalar(x_45)) { - x_50 = lean_alloc_ctor(0, 2, 0); -} else { - x_50 = x_45; +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Lean_Elab_Command_withCtorRef___rarg), 5, 0); +return x_3; } -lean_ctor_set(x_50, 0, x_43); -lean_ctor_set(x_50, 1, x_48); -x_51 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_51, 0, x_50); -lean_ctor_set(x_51, 1, x_3); -x_2 = x_42; -x_3 = x_51; -x_10 = x_49; -goto _start; } -else +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: { -lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; -lean_dec(x_45); -lean_dec(x_43); -lean_dec(x_42); +size_t x_11; size_t x_12; lean_object* x_13; +x_11 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_12 = lean_unbox_usize(x_9); lean_dec(x_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_53 = lean_ctor_get(x_47, 0); -lean_inc(x_53); -x_54 = lean_ctor_get(x_47, 1); -lean_inc(x_54); -if (lean_is_exclusive(x_47)) { - lean_ctor_release(x_47, 0); - lean_ctor_release(x_47, 1); - x_55 = x_47; -} else { - lean_dec_ref(x_47); - x_55 = lean_box(0); -} -if (lean_is_scalar(x_55)) { - x_56 = lean_alloc_ctor(1, 2, 0); -} else { - x_56 = x_55; +x_13 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg___lambda__1(x_1, x_11, x_3, x_4, x_5, x_6, x_7, x_8, x_12, x_10); +return x_13; } -lean_ctor_set(x_56, 0, x_53); -lean_ctor_set(x_56, 1, x_54); -return x_56; } +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___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_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg___lambda__2(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; } } +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg___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_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg___lambda__3(x_1, x_2, x_3, x_4); +lean_dec(x_4); +lean_dec(x_1); +return x_5; } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateParams___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_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___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) { _start: { -if (lean_obj_tag(x_2) == 0) -{ -lean_object* x_11; lean_object* x_12; -lean_dec(x_9); +size_t x_11; size_t x_12; lean_object* x_13; +x_11 = lean_unbox_usize(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_1); -x_11 = l_List_reverse___rarg(x_3); -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; +x_12 = lean_unbox_usize(x_9); +lean_dec(x_9); +x_13 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_11, x_12, x_10); +return x_13; } -else -{ -uint8_t x_13; -x_13 = !lean_is_exclusive(x_2); -if (x_13 == 0) -{ -lean_object* x_14; uint8_t x_15; -x_14 = lean_ctor_get(x_2, 0); -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; uint8_t x_20; uint8_t x_21; uint8_t x_22; lean_object* x_23; -x_16 = lean_ctor_get(x_2, 1); -x_17 = lean_ctor_get(x_14, 0); -x_18 = lean_ctor_get(x_14, 1); -x_19 = lean_ctor_get(x_14, 2); -x_20 = 0; -x_21 = 1; -x_22 = 1; -lean_inc(x_1); -x_23 = l_Lean_Meta_mkForallFVars(x_1, x_18, x_20, x_21, x_22, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_23) == 0) -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_23, 1); -lean_inc(x_25); -lean_dec(x_23); -x_26 = lean_box(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); -lean_inc(x_1); -x_27 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateParams___spec__1(x_1, x_19, x_26, x_4, x_5, x_6, x_7, x_8, x_9, x_25); -if (lean_obj_tag(x_27) == 0) -{ -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); -lean_ctor_set(x_14, 2, x_28); -lean_ctor_set(x_14, 1, x_24); -lean_ctor_set(x_2, 1, x_3); +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___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* _tmp_1 = x_16; -lean_object* _tmp_2 = x_2; -lean_object* _tmp_9 = x_29; -x_2 = _tmp_1; -x_3 = _tmp_2; -x_10 = _tmp_9; +size_t x_11; size_t x_12; lean_object* x_13; +x_11 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_12 = lean_unbox_usize(x_9); +lean_dec(x_9); +x_13 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__2___rarg___lambda__2(x_1, x_11, x_3, x_4, x_5, x_6, x_7, x_8, x_12, x_10); +return x_13; } -goto _start; } -else +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__2___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: { -uint8_t x_31; -lean_dec(x_24); -lean_free_object(x_14); -lean_dec(x_17); -lean_free_object(x_2); -lean_dec(x_16); -lean_dec(x_9); +size_t x_11; size_t x_12; lean_object* x_13; +x_11 = lean_unbox_usize(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_1); -x_31 = !lean_is_exclusive(x_27); -if (x_31 == 0) -{ -return x_27; +x_12 = lean_unbox_usize(x_9); +lean_dec(x_9); +x_13 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_withCtorRef___spec__2___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_11, x_12, x_10); +return x_13; } -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; } +LEAN_EXPORT lean_object* l_Lean_Elab_Command_withCtorRef___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Lean_Elab_Command_withCtorRef___rarg___lambda__1(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +return x_3; } } -else +LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +_start: { -uint8_t x_35; -lean_free_object(x_14); -lean_dec(x_19); -lean_dec(x_17); -lean_free_object(x_2); -lean_dec(x_16); +uint8_t x_16; +x_16 = lean_usize_dec_lt(x_6, x_5); +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_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_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; -} -} +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_7); +lean_ctor_set(x_17, 1, x_15); +return x_17; } else { -lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; uint8_t x_44; uint8_t x_45; lean_object* x_46; -x_39 = lean_ctor_get(x_2, 1); -x_40 = lean_ctor_get(x_14, 0); -x_41 = lean_ctor_get(x_14, 1); -x_42 = lean_ctor_get(x_14, 2); -lean_inc(x_42); -lean_inc(x_41); -lean_inc(x_40); -lean_dec(x_14); -x_43 = 0; -x_44 = 1; -x_45 = 1; -lean_inc(x_1); -x_46 = l_Lean_Meta_mkForallFVars(x_1, x_41, x_43, x_44, x_45, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_46) == 0) -{ -lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; -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_box(0); +lean_object* x_18; lean_object* x_19; lean_object* x_20; +lean_dec(x_7); +x_18 = lean_ctor_get(x_4, 0); +x_19 = lean_array_uget(x_18, x_6); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); +lean_inc(x_2); lean_inc(x_1); -x_50 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateParams___spec__1(x_1, x_42, x_49, x_4, x_5, x_6, x_7, x_8, x_9, x_48); -if (lean_obj_tag(x_50) == 0) -{ -lean_object* x_51; lean_object* x_52; lean_object* x_53; -x_51 = lean_ctor_get(x_50, 0); -lean_inc(x_51); -x_52 = lean_ctor_get(x_50, 1); -lean_inc(x_52); -lean_dec(x_50); -x_53 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_53, 0, x_40); -lean_ctor_set(x_53, 1, x_47); -lean_ctor_set(x_53, 2, x_51); -lean_ctor_set(x_2, 1, x_3); -lean_ctor_set(x_2, 0, x_53); +lean_inc(x_3); +x_20 = l_Lean_Elab_Command_accLevelAtCtor(x_3, x_19, x_1, x_2, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_20) == 0) { -lean_object* _tmp_1 = x_39; -lean_object* _tmp_2 = x_2; -lean_object* _tmp_9 = x_52; -x_2 = _tmp_1; -x_3 = _tmp_2; -x_10 = _tmp_9; -} +lean_object* x_21; size_t x_22; size_t x_23; lean_object* x_24; +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +x_22 = 1; +x_23 = lean_usize_add(x_6, x_22); +x_24 = lean_box(0); +x_6 = x_23; +x_7 = x_24; +x_15 = x_21; goto _start; } else { -lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; -lean_dec(x_47); -lean_dec(x_40); -lean_free_object(x_2); -lean_dec(x_39); +uint8_t x_26; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); lean_dec(x_3); +lean_dec(x_2); lean_dec(x_1); -x_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; -} +x_26 = !lean_is_exclusive(x_20); +if (x_26 == 0) +{ +return x_20; } else { -lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; -lean_dec(x_42); -lean_dec(x_40); -lean_free_object(x_2); -lean_dec(x_39); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_59 = lean_ctor_get(x_46, 0); -lean_inc(x_59); -x_60 = lean_ctor_get(x_46, 1); -lean_inc(x_60); -if (lean_is_exclusive(x_46)) { - lean_ctor_release(x_46, 0); - lean_ctor_release(x_46, 1); - x_61 = x_46; -} else { - lean_dec_ref(x_46); - x_61 = lean_box(0); +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_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; } -if (lean_is_scalar(x_61)) { - x_62 = lean_alloc_ctor(1, 2, 0); -} else { - x_62 = x_61; } -lean_ctor_set(x_62, 0, x_59); -lean_ctor_set(x_62, 1, x_60); -return x_62; } } } -else +LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___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, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_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; uint8_t x_69; uint8_t x_70; uint8_t x_71; lean_object* x_72; -x_63 = lean_ctor_get(x_2, 0); -x_64 = lean_ctor_get(x_2, 1); -lean_inc(x_64); -lean_inc(x_63); -lean_dec(x_2); -x_65 = lean_ctor_get(x_63, 0); -lean_inc(x_65); -x_66 = lean_ctor_get(x_63, 1); -lean_inc(x_66); -x_67 = lean_ctor_get(x_63, 2); -lean_inc(x_67); -if (lean_is_exclusive(x_63)) { - lean_ctor_release(x_63, 0); - lean_ctor_release(x_63, 1); - lean_ctor_release(x_63, 2); - x_68 = x_63; -} else { - lean_dec_ref(x_63); - x_68 = lean_box(0); +lean_object* x_12; +x_12 = lean_apply_10(x_1, x_5, x_6, x_2, x_3, x_4, x_7, x_8, x_9, x_10, x_11); +return x_12; } -x_69 = 0; -x_70 = 1; -x_71 = 1; -lean_inc(x_1); -x_72 = l_Lean_Meta_mkForallFVars(x_1, x_66, x_69, x_70, x_71, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_72) == 0) +} +LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__2___rarg(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_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; -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_box(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); -lean_inc(x_1); -x_76 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateParams___spec__1(x_1, x_67, x_75, x_4, x_5, x_6, x_7, x_8, x_9, x_74); -if (lean_obj_tag(x_76) == 0) +lean_object* x_12; lean_object* x_13; +x_12 = lean_alloc_closure((void*)(l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__2___rarg___lambda__1), 11, 4); +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_6); +x_13 = l___private_Lean_Meta_Basic_0__Lean_Meta_forallTelescopeReducingImp___rarg(x_1, x_12, x_3, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_13) == 0) { -lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; -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); -if (lean_is_scalar(x_68)) { - x_79 = lean_alloc_ctor(0, 3, 0); -} else { - x_79 = x_68; -} -lean_ctor_set(x_79, 0, x_65); -lean_ctor_set(x_79, 1, x_73); -lean_ctor_set(x_79, 2, x_77); -x_80 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_80, 0, x_79); -lean_ctor_set(x_80, 1, x_3); -x_2 = x_64; -x_3 = x_80; -x_10 = x_78; -goto _start; +uint8_t x_14; +x_14 = !lean_is_exclusive(x_13); +if (x_14 == 0) +{ +return x_13; } else { -lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; -lean_dec(x_73); -lean_dec(x_68); -lean_dec(x_65); -lean_dec(x_64); -lean_dec(x_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_82 = lean_ctor_get(x_76, 0); -lean_inc(x_82); -x_83 = lean_ctor_get(x_76, 1); -lean_inc(x_83); -if (lean_is_exclusive(x_76)) { - lean_ctor_release(x_76, 0); - lean_ctor_release(x_76, 1); - 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(1, 2, 0); -} else { - x_85 = x_84; -} -lean_ctor_set(x_85, 0, x_82); -lean_ctor_set(x_85, 1, x_83); -return x_85; +lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_15 = lean_ctor_get(x_13, 0); +x_16 = lean_ctor_get(x_13, 1); +lean_inc(x_16); +lean_inc(x_15); +lean_dec(x_13); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_15); +lean_ctor_set(x_17, 1, x_16); +return x_17; } } else { -lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; -lean_dec(x_68); -lean_dec(x_67); -lean_dec(x_65); -lean_dec(x_64); -lean_dec(x_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_86 = lean_ctor_get(x_72, 0); -lean_inc(x_86); -x_87 = lean_ctor_get(x_72, 1); -lean_inc(x_87); -if (lean_is_exclusive(x_72)) { - lean_ctor_release(x_72, 0); - lean_ctor_release(x_72, 1); - x_88 = x_72; -} else { - lean_dec_ref(x_72); - x_88 = lean_box(0); -} -if (lean_is_scalar(x_88)) { - x_89 = lean_alloc_ctor(1, 2, 0); -} else { - x_89 = x_88; -} -lean_ctor_set(x_89, 0, x_86); -lean_ctor_set(x_89, 1, x_87); -return x_89; +uint8_t x_18; +x_18 = !lean_is_exclusive(x_13); +if (x_18 == 0) +{ +return x_13; } +else +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_13, 0); +x_20 = lean_ctor_get(x_13, 1); +lean_inc(x_20); +lean_inc(x_19); +lean_dec(x_13); +x_21 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_21, 0, x_19); +lean_ctor_set(x_21, 1, x_20); +return x_21; } } } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateParams(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__2(lean_object* x_1) { _start: { -lean_object* x_10; lean_object* x_11; -x_10 = lean_box(0); -x_11 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateParams___spec__2(x_1, x_2, x_10, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_11; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__2___rarg___boxed), 11, 0); +return x_2; } } -LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectLevelParamsInInductive___spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { -if (lean_obj_tag(x_1) == 0) -{ -return x_2; -} -else +uint8_t x_16; +x_16 = lean_usize_dec_lt(x_6, x_5); +if (x_16 == 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); -x_4 = lean_ctor_get(x_1, 1); -lean_inc(x_4); -lean_dec(x_1); -x_5 = lean_ctor_get(x_3, 1); -lean_inc(x_5); +lean_object* x_17; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); lean_dec(x_3); -x_6 = l_Lean_CollectLevelParams_main(x_5, x_2); -x_1 = x_4; -x_2 = x_6; -goto _start; -} -} -} -LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectLevelParamsInInductive___spec__2(lean_object* x_1, lean_object* x_2) { -_start: -{ -if (lean_obj_tag(x_1) == 0) -{ -return x_2; +lean_dec(x_2); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_7); +lean_ctor_set(x_17, 1, x_15); +return x_17; } 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; -x_3 = lean_ctor_get(x_1, 0); +lean_object* x_18; lean_object* x_19; uint8_t x_20; +lean_dec(x_7); +x_18 = lean_array_uget(x_4, x_6); +x_19 = lean_ctor_get(x_18, 2); +lean_inc(x_19); +x_20 = lean_name_eq(x_19, x_1); +lean_dec(x_19); +if (x_20 == 0) +{ +size_t x_21; size_t x_22; +lean_dec(x_18); +x_21 = 1; +x_22 = lean_usize_add(x_6, x_21); lean_inc(x_3); -x_4 = lean_ctor_get(x_1, 1); -lean_inc(x_4); -lean_dec(x_1); -x_5 = lean_ctor_get(x_3, 1); -lean_inc(x_5); -x_6 = l_Lean_CollectLevelParams_main(x_5, x_2); -x_7 = lean_ctor_get(x_3, 2); -lean_inc(x_7); -lean_dec(x_3); -x_8 = l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectLevelParamsInInductive___spec__1(x_7, x_6); -x_1 = x_4; -x_2 = x_8; -goto _start; -} -} -} -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectLevelParamsInInductive___closed__1() { -_start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__2___closed__3; -x_2 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__3___closed__1; -x_3 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_1); -lean_ctor_set(x_3, 2, x_2); -return x_3; +size_t _tmp_5 = x_22; +lean_object* _tmp_6 = x_3; +x_6 = _tmp_5; +x_7 = _tmp_6; } +goto _start; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectLevelParamsInInductive(lean_object* x_1) { -_start: +else { -lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_2 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectLevelParamsInInductive___closed__1; -x_3 = l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectLevelParamsInInductive___spec__2(x_1, x_2); -x_4 = lean_ctor_get(x_3, 2); -lean_inc(x_4); +lean_object* x_24; uint8_t x_25; lean_dec(x_3); -return x_4; -} -} -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkIndFVar2Const___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -uint8_t x_11; -x_11 = lean_nat_dec_le(x_8, x_7); -if (x_11 == 0) +x_24 = lean_ctor_get(x_18, 0); +lean_inc(x_24); +lean_dec(x_18); +x_25 = !lean_is_exclusive(x_13); +if (x_25 == 0) { -lean_object* x_12; uint8_t x_13; -x_12 = lean_unsigned_to_nat(0u); -x_13 = lean_nat_dec_eq(x_6, x_12); -if (x_13 == 0) +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_13, 5); +x_27 = l_Lean_replaceRef(x_24, x_26); +lean_dec(x_26); +lean_dec(x_24); +lean_ctor_set(x_13, 5, x_27); +x_28 = lean_apply_8(x_2, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_28) == 0) { -lean_object* x_14; lean_object* x_15; uint8_t x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; -x_14 = lean_unsigned_to_nat(1u); -x_15 = lean_nat_sub(x_6, x_14); -lean_dec(x_6); -x_16 = lean_nat_dec_lt(x_7, x_5); -x_17 = lean_array_get_size(x_2); -x_18 = lean_nat_dec_lt(x_7, x_17); -lean_dec(x_17); -if (x_16 == 0) +uint8_t x_29; +x_29 = !lean_is_exclusive(x_28); +if (x_29 == 0) { -lean_object* x_71; lean_object* x_72; -x_71 = l_Lean_Elab_Command_instInhabitedInductiveView; -x_72 = l_outOfBounds___rarg(x_71); -x_19 = x_72; -goto block_70; +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_30 = lean_ctor_get(x_28, 0); +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_28, 0, x_33); +return x_28; } else { -lean_object* x_73; -x_73 = lean_array_fget(x_1, x_7); -x_19 = x_73; -goto block_70; +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_34 = lean_ctor_get(x_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, 1, 0); +lean_ctor_set(x_36, 0, x_34); +x_37 = lean_box(0); +x_38 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_38, 0, x_36); +lean_ctor_set(x_38, 1, x_37); +x_39 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_39, 0, x_38); +lean_ctor_set(x_39, 1, x_35); +return x_39; } -block_70: -{ -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, 4); -lean_inc(x_20); -lean_dec(x_19); -lean_inc(x_3); -x_21 = l_Lean_Expr_const___override(x_20, x_3); -if (x_18 == 0) -{ -lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_63 = l_Lean_instInhabitedExpr; -x_64 = l_outOfBounds___rarg(x_63); -x_65 = lean_ctor_get(x_10, 0); -lean_inc(x_65); -x_66 = lean_ctor_get(x_10, 1); -lean_inc(x_66); -lean_dec(x_10); -x_22 = x_64; -x_23 = x_65; -x_24 = x_66; -goto block_62; } else { -lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_67 = lean_array_fget(x_2, x_7); -x_68 = lean_ctor_get(x_10, 0); -lean_inc(x_68); -x_69 = lean_ctor_get(x_10, 1); -lean_inc(x_69); -lean_dec(x_10); -x_22 = x_67; -x_23 = x_68; -x_24 = x_69; -goto block_62; -} -block_62: -{ -lean_object* x_25; uint64_t x_26; uint64_t x_27; uint64_t x_28; uint64_t x_29; uint64_t x_30; uint64_t x_31; uint64_t x_32; size_t x_33; size_t x_34; size_t x_35; size_t x_36; size_t x_37; lean_object* x_38; uint8_t x_39; -x_25 = lean_array_get_size(x_24); -x_26 = l_Lean_Expr_hash(x_22); -x_27 = 32; -x_28 = lean_uint64_shift_right(x_26, x_27); -x_29 = lean_uint64_xor(x_26, x_28); -x_30 = 16; -x_31 = lean_uint64_shift_right(x_29, x_30); -x_32 = lean_uint64_xor(x_29, x_31); -x_33 = lean_uint64_to_usize(x_32); -x_34 = lean_usize_of_nat(x_25); -lean_dec(x_25); -x_35 = 1; -x_36 = lean_usize_sub(x_34, x_35); -x_37 = lean_usize_land(x_33, x_36); -x_38 = lean_array_uget(x_24, x_37); -x_39 = l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Elab_DeclNameGen_0__Lean_Elab_Command_NameGen_winnowExpr_visit___spec__1(x_22, x_38); -if (x_39 == 0) -{ -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; -x_40 = lean_nat_add(x_23, x_14); -lean_dec(x_23); -x_41 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_41, 0, x_22); -lean_ctor_set(x_41, 1, x_21); -lean_ctor_set(x_41, 2, x_38); -x_42 = lean_array_uset(x_24, x_37, x_41); -x_43 = lean_unsigned_to_nat(4u); -x_44 = lean_nat_mul(x_40, x_43); -x_45 = lean_unsigned_to_nat(3u); -x_46 = lean_nat_div(x_44, x_45); -lean_dec(x_44); -x_47 = lean_array_get_size(x_42); -x_48 = lean_nat_dec_le(x_46, x_47); -lean_dec(x_47); -lean_dec(x_46); -if (x_48 == 0) +uint8_t x_40; +x_40 = !lean_is_exclusive(x_28); +if (x_40 == 0) { -lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_49 = l_Std_DHashMap_Internal_Raw_u2080_expand___at___private_Lean_Elab_DeclNameGen_0__Lean_Elab_Command_NameGen_winnowExpr_visit___spec__2(x_42); -x_50 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_50, 0, x_40); -lean_ctor_set(x_50, 1, x_49); -x_51 = lean_nat_add(x_7, x_9); -lean_dec(x_7); -x_6 = x_15; -x_7 = x_51; -x_10 = x_50; -goto _start; +return x_28; } else { -lean_object* x_53; lean_object* x_54; -x_53 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_53, 0, x_40); -lean_ctor_set(x_53, 1, x_42); -x_54 = lean_nat_add(x_7, x_9); -lean_dec(x_7); -x_6 = x_15; -x_7 = x_54; -x_10 = x_53; -goto _start; +lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_41 = lean_ctor_get(x_28, 0); +x_42 = lean_ctor_get(x_28, 1); +lean_inc(x_42); +lean_inc(x_41); +lean_dec(x_28); +x_43 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_43, 0, x_41); +lean_ctor_set(x_43, 1, x_42); +return x_43; +} } } else { -lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; -lean_inc(x_4); -x_56 = lean_array_uset(x_24, x_37, x_4); -x_57 = l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Elab_DeclNameGen_0__Lean_Elab_Command_NameGen_winnowExpr_visit___spec__5(x_22, x_21, x_38); -x_58 = lean_array_uset(x_56, x_37, x_57); -x_59 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_59, 0, x_23); -lean_ctor_set(x_59, 1, x_58); -x_60 = lean_nat_add(x_7, x_9); -lean_dec(x_7); -x_6 = x_15; -x_7 = x_60; -x_10 = x_59; -goto _start; -} +lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; uint8_t x_55; lean_object* x_56; uint8_t x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; +x_44 = lean_ctor_get(x_13, 0); +x_45 = lean_ctor_get(x_13, 1); +x_46 = lean_ctor_get(x_13, 2); +x_47 = lean_ctor_get(x_13, 3); +x_48 = lean_ctor_get(x_13, 4); +x_49 = lean_ctor_get(x_13, 5); +x_50 = lean_ctor_get(x_13, 6); +x_51 = lean_ctor_get(x_13, 7); +x_52 = lean_ctor_get(x_13, 8); +x_53 = lean_ctor_get(x_13, 9); +x_54 = lean_ctor_get(x_13, 10); +x_55 = lean_ctor_get_uint8(x_13, sizeof(void*)*12); +x_56 = lean_ctor_get(x_13, 11); +x_57 = lean_ctor_get_uint8(x_13, sizeof(void*)*12 + 1); +lean_inc(x_56); +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_dec(x_13); +x_58 = l_Lean_replaceRef(x_24, x_49); +lean_dec(x_49); +lean_dec(x_24); +x_59 = lean_alloc_ctor(0, 12, 2); +lean_ctor_set(x_59, 0, x_44); +lean_ctor_set(x_59, 1, x_45); +lean_ctor_set(x_59, 2, x_46); +lean_ctor_set(x_59, 3, x_47); +lean_ctor_set(x_59, 4, x_48); +lean_ctor_set(x_59, 5, x_58); +lean_ctor_set(x_59, 6, x_50); +lean_ctor_set(x_59, 7, x_51); +lean_ctor_set(x_59, 8, x_52); +lean_ctor_set(x_59, 9, x_53); +lean_ctor_set(x_59, 10, x_54); +lean_ctor_set(x_59, 11, x_56); +lean_ctor_set_uint8(x_59, sizeof(void*)*12, x_55); +lean_ctor_set_uint8(x_59, sizeof(void*)*12 + 1, x_57); +x_60 = lean_apply_8(x_2, x_8, x_9, x_10, x_11, x_12, x_59, x_14, x_15); +if (lean_obj_tag(x_60) == 0) +{ +lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; +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); } +x_64 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_64, 0, x_61); +x_65 = lean_box(0); +x_66 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_66, 0, x_64); +lean_ctor_set(x_66, 1, x_65); +if (lean_is_scalar(x_63)) { + x_67 = lean_alloc_ctor(0, 2, 0); +} else { + x_67 = x_63; } +lean_ctor_set(x_67, 0, x_66); +lean_ctor_set(x_67, 1, x_62); +return x_67; } else { -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_4); -lean_dec(x_3); -return x_10; +lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; +x_68 = lean_ctor_get(x_60, 0); +lean_inc(x_68); +x_69 = lean_ctor_get(x_60, 1); +lean_inc(x_69); +if (lean_is_exclusive(x_60)) { + lean_ctor_release(x_60, 0); + lean_ctor_release(x_60, 1); + x_70 = x_60; +} else { + lean_dec_ref(x_60); + x_70 = lean_box(0); } +if (lean_is_scalar(x_70)) { + x_71 = lean_alloc_ctor(1, 2, 0); +} else { + x_71 = x_70; } -else -{ -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_4); -lean_dec(x_3); -return x_10; +lean_ctor_set(x_71, 0, x_68); +lean_ctor_set(x_71, 1, x_69); +return x_71; } } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkIndFVar2Const(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 = lean_box(0); -x_5 = l_List_mapTR_loop___at_Lean_mkConstWithLevelParams___spec__1(x_3, x_4); -x_6 = lean_box(0); -x_7 = lean_array_get_size(x_1); -x_8 = lean_unsigned_to_nat(0u); -x_9 = lean_unsigned_to_nat(1u); -x_10 = l_Lean_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__2___closed__3; -lean_inc(x_7); -x_11 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkIndFVar2Const___spec__1(x_1, x_2, x_5, x_6, x_7, x_7, x_8, x_7, x_9, x_10); -lean_dec(x_7); -return x_11; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkIndFVar2Const___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, 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_11; -x_11 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkIndFVar2Const___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +uint8_t x_16; +x_16 = lean_usize_dec_lt(x_6, x_5); +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_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_5); +lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -return x_11; -} +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_7); +lean_ctor_set(x_17, 1, x_15); +return x_17; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkIndFVar2Const___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: +else { -lean_object* x_4; -x_4 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkIndFVar2Const(x_1, x_2, x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_4; -} -} -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: +lean_object* x_18; lean_object* x_19; size_t x_20; size_t x_21; lean_object* x_22; +lean_dec(x_7); +x_18 = lean_array_uget(x_4, x_6); +x_19 = lean_ctor_get(x_18, 8); +lean_inc(x_19); +lean_dec(x_18); +x_20 = lean_array_size(x_19); +x_21 = 0; +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc_n(x_3, 2); +lean_inc(x_2); +x_22 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__4(x_1, x_2, x_3, x_19, x_20, x_21, x_3, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +lean_dec(x_19); +if (lean_obj_tag(x_22) == 0) { -uint8_t x_5; -x_5 = l_Lean_Expr_isFVar(x_4); -if (x_5 == 0) +lean_object* x_23; lean_object* x_24; +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +lean_dec(x_23); +if (lean_obj_tag(x_24) == 0) { -lean_object* x_6; -x_6 = lean_box(0); -return x_6; +lean_object* x_25; size_t x_26; size_t x_27; +x_25 = lean_ctor_get(x_22, 1); +lean_inc(x_25); +lean_dec(x_22); +x_26 = 1; +x_27 = lean_usize_add(x_6, x_26); +lean_inc(x_3); +{ +size_t _tmp_5 = x_27; +lean_object* _tmp_6 = x_3; +lean_object* _tmp_14 = x_25; +x_6 = _tmp_5; +x_7 = _tmp_6; +x_15 = _tmp_14; +} +goto _start; } else { -lean_object* x_7; lean_object* x_8; uint64_t x_9; uint64_t x_10; uint64_t x_11; uint64_t x_12; uint64_t x_13; uint64_t x_14; uint64_t x_15; size_t x_16; size_t x_17; size_t x_18; size_t x_19; size_t x_20; lean_object* x_21; lean_object* x_22; -x_7 = lean_ctor_get(x_1, 1); -x_8 = lean_array_get_size(x_7); -x_9 = l_Lean_Expr_hash(x_4); -x_10 = 32; -x_11 = lean_uint64_shift_right(x_9, x_10); -x_12 = lean_uint64_xor(x_9, x_11); -x_13 = 16; -x_14 = lean_uint64_shift_right(x_12, x_13); -x_15 = lean_uint64_xor(x_12, x_14); -x_16 = lean_uint64_to_usize(x_15); -x_17 = lean_usize_of_nat(x_8); -lean_dec(x_8); -x_18 = 1; -x_19 = lean_usize_sub(x_17, x_18); -x_20 = lean_usize_land(x_16, x_19); -x_21 = lean_array_uget(x_7, x_20); -x_22 = l_Std_DHashMap_Internal_AssocList_get_x3f___at___private_Lean_Elab_DeclNameGen_0__Lean_Elab_Command_NameGen_winnowExpr_visit___spec__6(x_4, x_21); -lean_dec(x_21); -if (lean_obj_tag(x_22) == 0) +uint8_t x_29; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_3); +lean_dec(x_2); +x_29 = !lean_is_exclusive(x_22); +if (x_29 == 0) { -lean_object* x_23; -x_23 = lean_box(0); -return x_23; +lean_object* x_30; uint8_t x_31; +x_30 = lean_ctor_get(x_22, 0); +lean_dec(x_30); +x_31 = !lean_is_exclusive(x_24); +if (x_31 == 0) +{ +lean_object* x_32; lean_object* x_33; +x_32 = lean_box(0); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_24); +lean_ctor_set(x_33, 1, x_32); +lean_ctor_set(x_22, 0, x_33); +return x_22; } else { -uint8_t x_24; -x_24 = !lean_is_exclusive(x_22); -if (x_24 == 0) +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_34 = lean_ctor_get(x_24, 0); +lean_inc(x_34); +lean_dec(x_24); +x_35 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_35, 0, x_34); +x_36 = lean_box(0); +x_37 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +lean_ctor_set(x_22, 0, x_37); +return x_22; +} +} +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; +x_38 = lean_ctor_get(x_22, 1); +lean_inc(x_38); +lean_dec(x_22); +x_39 = lean_ctor_get(x_24, 0); +lean_inc(x_39); +if (lean_is_exclusive(x_24)) { + lean_ctor_release(x_24, 0); + x_40 = x_24; +} else { + lean_dec_ref(x_24); + 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_box(0); +x_43 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_43, 0, x_41); +lean_ctor_set(x_43, 1, x_42); +x_44 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_44, 0, x_43); +lean_ctor_set(x_44, 1, x_38); +return x_44; +} +} +} +else +{ +uint8_t x_45; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_3); +lean_dec(x_2); +x_45 = !lean_is_exclusive(x_22); +if (x_45 == 0) { -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_25 = lean_ctor_get(x_22, 0); -x_26 = lean_unsigned_to_nat(0u); -x_27 = l_Array_extract___rarg(x_2, x_26, x_3); -x_28 = l_Lean_mkAppN(x_25, x_27); -lean_dec(x_27); -lean_ctor_set(x_22, 0, x_28); return x_22; } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_29 = lean_ctor_get(x_22, 0); -lean_inc(x_29); +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_30 = lean_unsigned_to_nat(0u); -x_31 = l_Array_extract___rarg(x_2, x_30, x_3); -x_32 = l_Lean_mkAppN(x_29, x_31); -lean_dec(x_31); -x_33 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_33, 0, x_32); -return x_33; +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_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___spec__1___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_withCtorRef___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__3___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_12; lean_object* x_13; uint8_t x_14; uint8_t x_15; uint8_t x_16; lean_object* x_17; +lean_object* x_11; +x_11 = lean_apply_8(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_withCtorRef___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___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: +{ +size_t x_12; size_t x_13; lean_object* x_14; lean_object* x_15; +x_12 = lean_array_size(x_1); +x_13 = 0; +x_14 = l_Lean_Elab_Command_withCtorRef___rarg___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_4); lean_inc(x_3); -x_12 = lean_alloc_closure((void*)(l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___spec__1___lambda__1___boxed), 4, 3); -lean_closure_set(x_12, 0, x_1); -lean_closure_set(x_12, 1, x_3); -lean_closure_set(x_12, 2, x_2); -x_13 = lean_replace_expr(x_12, x_4); -lean_dec(x_12); -x_14 = 0; -x_15 = 1; -x_16 = 1; -x_17 = l_Lean_Meta_mkForallFVars(x_3, x_13, x_14, x_15, x_16, x_7, x_8, x_9, x_10, x_11); +x_15 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__5(x_2, x_3, x_14, x_1, x_12, x_13, x_14, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_15) == 0) +{ +lean_object* x_16; lean_object* x_17; +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +lean_dec(x_16); 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_object* x_18; lean_object* x_19; +x_18 = lean_ctor_get(x_15, 1); lean_inc(x_18); -x_19 = lean_ctor_get(x_17, 1); -lean_inc(x_19); -lean_dec(x_17); -x_20 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_19); -return x_20; +lean_dec(x_15); +x_19 = lean_apply_8(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_18); +return x_19; } else { -uint8_t x_21; -x_21 = !lean_is_exclusive(x_17); -if (x_21 == 0) +uint8_t x_20; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_20 = !lean_is_exclusive(x_15); +if (x_20 == 0) { -return x_17; +lean_object* x_21; lean_object* x_22; +x_21 = lean_ctor_get(x_15, 0); +lean_dec(x_21); +x_22 = lean_ctor_get(x_17, 0); +lean_inc(x_22); +lean_dec(x_17); +lean_ctor_set(x_15, 0, x_22); +return x_15; } 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_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_15, 1); lean_inc(x_23); -lean_inc(x_22); +lean_dec(x_15); +x_24 = lean_ctor_get(x_17, 0); +lean_inc(x_24); 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; +x_25 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_25, 0, x_24); +lean_ctor_set(x_25, 1, x_23); +return x_25; +} +} +} +else +{ +uint8_t x_26; +lean_dec(x_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 = !lean_is_exclusive(x_15); +if (x_26 == 0) +{ +return x_15; +} +else +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_15, 0); +x_28 = lean_ctor_get(x_15, 1); +lean_inc(x_28); +lean_inc(x_27); +lean_dec(x_15); +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_27); +lean_ctor_set(x_29, 1, x_28); +return x_29; } } } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___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_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___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, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { -if (lean_obj_tag(x_4) == 0) +lean_object* x_15; lean_object* x_16; lean_object* x_17; size_t x_18; lean_object* x_19; size_t x_20; lean_object* x_21; lean_object* x_22; +x_15 = lean_array_get_size(x_5); +x_16 = l_Array_toSubarray___rarg(x_5, x_1, x_15); +x_17 = lean_ctor_get(x_16, 2); +lean_inc(x_17); +x_18 = lean_usize_of_nat(x_17); +lean_dec(x_17); +x_19 = lean_ctor_get(x_16, 1); +lean_inc(x_19); +x_20 = lean_usize_of_nat(x_19); +lean_dec(x_19); +x_21 = lean_box(0); +x_22 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__1(x_2, x_3, x_4, x_16, x_18, x_20, x_21, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_16); +if (lean_obj_tag(x_22) == 0) { -lean_object* x_13; lean_object* x_14; +uint8_t x_23; +x_23 = !lean_is_exclusive(x_22); +if (x_23 == 0) +{ +lean_object* x_24; +x_24 = lean_ctor_get(x_22, 0); +lean_dec(x_24); +lean_ctor_set(x_22, 0, x_21); +return x_22; +} +else +{ +lean_object* x_25; lean_object* x_26; +x_25 = lean_ctor_get(x_22, 1); +lean_inc(x_25); +lean_dec(x_22); +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_21); +lean_ctor_set(x_26, 1, x_25); +return x_26; +} +} +else +{ +uint8_t x_27; +x_27 = !lean_is_exclusive(x_22); +if (x_27 == 0) +{ +return x_22; +} +else +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_22, 0); +x_29 = lean_ctor_get(x_22, 1); +lean_inc(x_29); +lean_inc(x_28); +lean_dec(x_22); +x_30 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_14; lean_object* x_15; +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_13 = l_List_reverse___rarg(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; +x_14 = lean_box(0); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_13); +return x_15; } else { -uint8_t x_15; -x_15 = !lean_is_exclusive(x_4); -if (x_15 == 0) -{ -lean_object* x_16; uint8_t x_17; -x_16 = lean_ctor_get(x_4, 0); -x_17 = !lean_is_exclusive(x_16); -if (x_17 == 0) -{ -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; lean_object* x_24; -x_18 = lean_ctor_get(x_4, 1); -x_19 = lean_ctor_get(x_16, 0); -x_20 = lean_ctor_get(x_16, 1); -lean_inc(x_2); -x_21 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_21, 0, x_2); -lean_inc(x_1); +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_16 = lean_ctor_get(x_5, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_5, 1); +lean_inc(x_17); +lean_dec(x_5); +x_18 = lean_ctor_get(x_16, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_16, 1); +lean_inc(x_19); lean_inc(x_3); -x_22 = lean_alloc_closure((void*)(l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___spec__1___lambda__2___boxed), 11, 2); -lean_closure_set(x_22, 0, x_3); -lean_closure_set(x_22, 1, x_1); -x_23 = 0; +lean_inc(x_2); +lean_inc(x_4); +x_20 = lean_alloc_closure((void*)(l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__6___lambda__1___boxed), 14, 4); +lean_closure_set(x_20, 0, x_4); +lean_closure_set(x_20, 1, x_2); +lean_closure_set(x_20, 2, x_3); +lean_closure_set(x_20, 3, x_16); +x_21 = 0; +x_22 = lean_box(x_21); +x_23 = lean_alloc_closure((void*)(l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__2___rarg___boxed), 11, 3); +lean_closure_set(x_23, 0, x_19); +lean_closure_set(x_23, 1, x_20); +lean_closure_set(x_23, 2, x_22); +lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -x_24 = l_Lean_Meta_forallBoundedTelescope___at_Lean_Elab_Term_addAutoBoundImplicits_x27___spec__2___rarg(x_20, x_21, x_22, x_23, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_24 = l_Lean_Elab_Command_withCtorRef___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__3(x_1, x_18, x_23, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_18); if (lean_obj_tag(x_24) == 0) { -lean_object* x_25; lean_object* x_26; -x_25 = lean_ctor_get(x_24, 0); +lean_object* x_25; +x_25 = lean_ctor_get(x_24, 1); lean_inc(x_25); -x_26 = lean_ctor_get(x_24, 1); -lean_inc(x_26); lean_dec(x_24); -lean_ctor_set(x_16, 1, x_25); -lean_ctor_set(x_4, 1, x_5); -{ -lean_object* _tmp_3 = x_18; -lean_object* _tmp_4 = x_4; -lean_object* _tmp_11 = x_26; -x_4 = _tmp_3; -x_5 = _tmp_4; -x_12 = _tmp_11; -} +x_5 = x_17; +x_13 = x_25; goto _start; } else { -uint8_t x_28; -lean_free_object(x_16); -lean_dec(x_19); -lean_free_object(x_4); -lean_dec(x_18); +uint8_t x_27; +lean_dec(x_17); +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_28 = !lean_is_exclusive(x_24); -if (x_28 == 0) +x_27 = !lean_is_exclusive(x_24); +if (x_27 == 0) { return x_24; } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_24, 0); -x_30 = lean_ctor_get(x_24, 1); -lean_inc(x_30); +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_24, 0); +x_29 = lean_ctor_get(x_24, 1); lean_inc(x_29); +lean_inc(x_28); 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; +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_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_14; lean_object* x_15; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_14 = lean_box(0); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_13); +return x_15; } else { -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; lean_object* x_38; -x_32 = lean_ctor_get(x_4, 1); -x_33 = lean_ctor_get(x_16, 0); -x_34 = lean_ctor_get(x_16, 1); -lean_inc(x_34); -lean_inc(x_33); +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_16 = lean_ctor_get(x_5, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_5, 1); +lean_inc(x_17); +lean_dec(x_5); +x_18 = lean_ctor_get(x_16, 2); +lean_inc(x_18); lean_dec(x_16); -lean_inc(x_2); -x_35 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_35, 0, x_2); -lean_inc(x_1); -lean_inc(x_3); -x_36 = lean_alloc_closure((void*)(l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___spec__1___lambda__2___boxed), 11, 2); -lean_closure_set(x_36, 0, x_3); -lean_closure_set(x_36, 1, x_1); -x_37 = 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); lean_inc(x_6); -x_38 = l_Lean_Meta_forallBoundedTelescope___at_Lean_Elab_Term_addAutoBoundImplicits_x27___spec__2___rarg(x_34, x_35, x_36, x_37, 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; -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_alloc_ctor(0, 2, 0); -lean_ctor_set(x_41, 0, x_33); -lean_ctor_set(x_41, 1, x_39); -lean_ctor_set(x_4, 1, x_5); -lean_ctor_set(x_4, 0, x_41); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +x_19 = l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__6(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); +if (lean_obj_tag(x_19) == 0) { -lean_object* _tmp_3 = x_32; -lean_object* _tmp_4 = x_4; -lean_object* _tmp_11 = x_40; -x_4 = _tmp_3; -x_5 = _tmp_4; -x_12 = _tmp_11; -} +lean_object* x_20; +x_20 = lean_ctor_get(x_19, 1); +lean_inc(x_20); +lean_dec(x_19); +x_5 = x_17; +x_13 = x_20; goto _start; } else { -lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; -lean_dec(x_33); -lean_free_object(x_4); -lean_dec(x_32); +uint8_t x_22; +lean_dec(x_17); +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_43 = lean_ctor_get(x_38, 0); -lean_inc(x_43); -x_44 = lean_ctor_get(x_38, 1); -lean_inc(x_44); -if (lean_is_exclusive(x_38)) { - lean_ctor_release(x_38, 0); - lean_ctor_release(x_38, 1); - x_45 = x_38; -} else { - lean_dec_ref(x_38); - x_45 = lean_box(0); +x_22 = !lean_is_exclusive(x_19); +if (x_22 == 0) +{ +return x_19; } -if (lean_is_scalar(x_45)) { - x_46 = lean_alloc_ctor(1, 2, 0); -} else { - x_46 = x_45; +else +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_19, 0); +x_24 = lean_ctor_get(x_19, 1); +lean_inc(x_24); +lean_inc(x_23); +lean_dec(x_19); +x_25 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +return x_25; } -lean_ctor_set(x_46, 0, x_43); -lean_ctor_set(x_46, 1, x_44); -return x_46; } } } -else +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: { -lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; uint8_t x_54; lean_object* x_55; -x_47 = lean_ctor_get(x_4, 0); -x_48 = lean_ctor_get(x_4, 1); -lean_inc(x_48); -lean_inc(x_47); +lean_object* x_14; +x_14 = l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___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); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +_start: +{ +size_t x_16; size_t x_17; lean_object* x_18; +x_16 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_17 = lean_unbox_usize(x_6); +lean_dec(x_6); +x_18 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__1(x_1, x_2, x_3, x_4, x_16, x_17, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); lean_dec(x_4); -x_49 = lean_ctor_get(x_47, 0); -lean_inc(x_49); -x_50 = lean_ctor_get(x_47, 1); -lean_inc(x_50); -if (lean_is_exclusive(x_47)) { - lean_ctor_release(x_47, 0); - lean_ctor_release(x_47, 1); - x_51 = x_47; -} else { - lean_dec_ref(x_47); - x_51 = lean_box(0); +return x_18; } -lean_inc(x_2); -x_52 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_52, 0, x_2); -lean_inc(x_1); -lean_inc(x_3); -x_53 = lean_alloc_closure((void*)(l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___spec__1___lambda__2___boxed), 11, 2); -lean_closure_set(x_53, 0, x_3); -lean_closure_set(x_53, 1, x_1); -x_54 = 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_55 = l_Lean_Meta_forallBoundedTelescope___at_Lean_Elab_Term_addAutoBoundImplicits_x27___spec__2___rarg(x_50, x_52, x_53, x_54, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_55) == 0) +} +LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__2___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: { -lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; -x_56 = lean_ctor_get(x_55, 0); -lean_inc(x_56); -x_57 = lean_ctor_get(x_55, 1); -lean_inc(x_57); -lean_dec(x_55); -if (lean_is_scalar(x_51)) { - x_58 = lean_alloc_ctor(0, 2, 0); -} else { - x_58 = x_51; +uint8_t x_12; lean_object* x_13; +x_12 = lean_unbox(x_3); +lean_dec(x_3); +x_13 = l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__2___rarg(x_1, x_2, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_13; } -lean_ctor_set(x_58, 0, x_49); -lean_ctor_set(x_58, 1, x_56); -x_59 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_59, 0, x_58); -lean_ctor_set(x_59, 1, x_5); -x_4 = x_48; -x_5 = x_59; -x_12 = x_57; -goto _start; } -else +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +_start: { -lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; -lean_dec(x_51); -lean_dec(x_49); -lean_dec(x_48); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); +size_t x_16; size_t x_17; lean_object* x_18; +x_16 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_17 = lean_unbox_usize(x_6); lean_dec(x_6); +x_18 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__4(x_1, x_2, x_3, x_4, x_16, x_17, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +lean_dec(x_4); +lean_dec(x_1); +return x_18; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +_start: +{ +size_t x_16; size_t x_17; lean_object* x_18; +x_16 = lean_unbox_usize(x_5); lean_dec(x_5); -lean_dec(x_3); -lean_dec(x_2); +x_17 = lean_unbox_usize(x_6); +lean_dec(x_6); +x_18 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__5(x_1, x_2, x_3, x_4, x_16, x_17, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +lean_dec(x_4); lean_dec(x_1); -x_61 = lean_ctor_get(x_55, 0); -lean_inc(x_61); -x_62 = lean_ctor_get(x_55, 1); -lean_inc(x_62); -if (lean_is_exclusive(x_55)) { - lean_ctor_release(x_55, 0); - lean_ctor_release(x_55, 1); - x_63 = x_55; -} else { - lean_dec_ref(x_55); - x_63 = lean_box(0); +return x_18; } -if (lean_is_scalar(x_63)) { - x_64 = lean_alloc_ctor(1, 2, 0); -} else { - x_64 = x_63; } -lean_ctor_set(x_64, 0, x_61); -lean_ctor_set(x_64, 1, x_62); -return x_64; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_withCtorRef___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__3___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_Elab_Command_withCtorRef___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__3___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_2); +return x_11; +} +} +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* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, 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_Command_withCtorRef___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_2); +lean_dec(x_1); +return x_12; +} } +LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___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_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; +x_15 = l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__6___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_6); +return x_15; } } +LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_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, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; +x_14 = l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_1); +return x_14; } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___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_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -if (lean_obj_tag(x_4) == 0) +lean_object* x_14; +x_14 = l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___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_1); +return x_14; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: { -lean_object* x_13; 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_3); -lean_dec(x_2); +lean_object* x_14; +x_14 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); lean_dec(x_1); -x_13 = l_List_reverse___rarg(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; } +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_13 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__8___closed__1; +x_14 = lean_st_mk_ref(x_13, x_12); +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); +lean_inc(x_15); +x_17 = l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__7(x_1, x_2, x_3, x_4, x_5, x_15, x_6, x_7, x_8, x_9, x_10, x_11, x_16); +if (lean_obj_tag(x_17) == 0) +{ +lean_object* x_18; lean_object* x_19; uint8_t x_20; +x_18 = lean_ctor_get(x_17, 1); +lean_inc(x_18); +lean_dec(x_17); +x_19 = lean_st_ref_get(x_15, x_18); +lean_dec(x_15); +x_20 = !lean_is_exclusive(x_19); +if (x_20 == 0) +{ +return x_19; +} else { -uint8_t x_15; -x_15 = !lean_is_exclusive(x_4); -if (x_15 == 0) +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_19, 0); +x_22 = lean_ctor_get(x_19, 1); +lean_inc(x_22); +lean_inc(x_21); +lean_dec(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); +return x_23; +} +} +else { -lean_object* x_16; uint8_t x_17; -x_16 = lean_ctor_get(x_4, 0); -x_17 = !lean_is_exclusive(x_16); -if (x_17 == 0) +uint8_t x_24; +lean_dec(x_15); +x_24 = !lean_is_exclusive(x_17); +if (x_24 == 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_4, 1); -x_19 = lean_ctor_get(x_16, 0); -x_20 = lean_ctor_get(x_16, 1); -x_21 = lean_ctor_get(x_16, 2); -x_22 = lean_box(0); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_3); -lean_inc(x_2); -lean_inc(x_1); -x_23 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___spec__1(x_1, x_2, x_3, x_21, x_22, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_23) == 0) +return x_17; +} +else { -lean_object* x_24; lean_object* x_25; -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_17, 0); +x_26 = lean_ctor_get(x_17, 1); +lean_inc(x_26); lean_inc(x_25); -lean_dec(x_23); -lean_ctor_set(x_16, 2, x_24); -lean_ctor_set(x_4, 1, x_5); +lean_dec(x_17); +x_27 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +return x_27; +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, 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* _tmp_3 = x_18; -lean_object* _tmp_4 = x_4; -lean_object* _tmp_11 = x_25; -x_4 = _tmp_3; -x_5 = _tmp_4; -x_12 = _tmp_11; +lean_object* x_13; +x_13 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_1); +return x_13; } -goto _start; } -else +LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___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) { +_start: { -uint8_t x_27; -lean_free_object(x_16); -lean_dec(x_20); -lean_dec(x_19); -lean_free_object(x_4); -lean_dec(x_18); -lean_dec(x_11); -lean_dec(x_10); +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = lean_array_get_size(x_2); +x_10 = lean_nat_sub(x_9, x_1); lean_dec(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_8); +return x_11; +} +} +static lean_object* _init_l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__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_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__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_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__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; +} +} +LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +if (lean_obj_tag(x_3) == 0) +{ +lean_object* 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_2); lean_dec(x_1); -x_27 = !lean_is_exclusive(x_23); -if (x_27 == 0) -{ -return x_23; -} -else -{ -lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_28 = lean_ctor_get(x_23, 0); -x_29 = lean_ctor_get(x_23, 1); -lean_inc(x_29); -lean_inc(x_28); -lean_dec(x_23); -x_30 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_30, 0, x_28); -lean_ctor_set(x_30, 1, x_29); -return x_30; -} -} +x_10 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_10, 0, x_4); +lean_ctor_set(x_10, 1, x_9); +return x_10; } else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_31 = lean_ctor_get(x_4, 1); -x_32 = lean_ctor_get(x_16, 0); -x_33 = lean_ctor_get(x_16, 1); -x_34 = lean_ctor_get(x_16, 2); -lean_inc(x_34); -lean_inc(x_33); -lean_inc(x_32); -lean_dec(x_16); -x_35 = lean_box(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_dec(x_4); +x_11 = lean_ctor_get(x_3, 0); lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); +x_12 = lean_ctor_get(x_3, 1); +lean_inc(x_12); +lean_dec(x_3); +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +lean_inc(x_1); +x_14 = lean_alloc_closure((void*)(l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__1___lambda__1___boxed), 8, 1); +lean_closure_set(x_14, 0, x_1); +x_15 = 0; lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -lean_inc(x_3); -lean_inc(x_2); -lean_inc(x_1); -x_36 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___spec__1(x_1, x_2, x_3, x_34, x_35, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_36) == 0) +lean_inc(x_5); +x_16 = l_Lean_Meta_forallTelescopeReducing___at_Lean_Meta_getParamNames___spec__2___rarg(x_13, x_14, x_15, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_16) == 0) { -lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_37 = lean_ctor_get(x_36, 0); -lean_inc(x_37); -x_38 = lean_ctor_get(x_36, 1); -lean_inc(x_38); -lean_dec(x_36); -x_39 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_39, 0, x_32); -lean_ctor_set(x_39, 1, x_33); -lean_ctor_set(x_39, 2, x_37); -lean_ctor_set(x_4, 1, x_5); -lean_ctor_set(x_4, 0, x_39); +uint8_t x_17; +x_17 = !lean_is_exclusive(x_16); +if (x_17 == 0) { -lean_object* _tmp_3 = x_31; -lean_object* _tmp_4 = x_4; -lean_object* _tmp_11 = x_38; +lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_18 = lean_ctor_get(x_16, 0); +x_19 = lean_ctor_get(x_16, 1); +x_20 = lean_unsigned_to_nat(0u); +x_21 = lean_nat_dec_eq(x_18, x_20); +lean_dec(x_18); +if (x_21 == 0) +{ +lean_object* x_22; +lean_dec(x_12); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +lean_dec(x_1); +x_22 = l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__1___closed__2; +lean_ctor_set(x_16, 0, x_22); +return x_16; +} +else +{ +lean_free_object(x_16); +lean_inc(x_2); +{ +lean_object* _tmp_2 = x_12; +lean_object* _tmp_3 = x_2; +lean_object* _tmp_8 = x_19; +x_3 = _tmp_2; x_4 = _tmp_3; -x_5 = _tmp_4; -x_12 = _tmp_11; +x_9 = _tmp_8; } goto _start; } +} else { -lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; -lean_dec(x_33); -lean_dec(x_32); -lean_free_object(x_4); -lean_dec(x_31); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); +lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; +x_24 = lean_ctor_get(x_16, 0); +x_25 = lean_ctor_get(x_16, 1); +lean_inc(x_25); +lean_inc(x_24); +lean_dec(x_16); +x_26 = lean_unsigned_to_nat(0u); +x_27 = lean_nat_dec_eq(x_24, x_26); +lean_dec(x_24); +if (x_27 == 0) +{ +lean_object* x_28; lean_object* x_29; +lean_dec(x_12); 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_41 = lean_ctor_get(x_36, 0); -lean_inc(x_41); -x_42 = lean_ctor_get(x_36, 1); -lean_inc(x_42); -if (lean_is_exclusive(x_36)) { - lean_ctor_release(x_36, 0); - lean_ctor_release(x_36, 1); - x_43 = x_36; -} else { - lean_dec_ref(x_36); - 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; -} -} +x_28 = l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__1___closed__2; +x_29 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_25); +return x_29; } else { -lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_45 = lean_ctor_get(x_4, 0); -x_46 = lean_ctor_get(x_4, 1); -lean_inc(x_46); -lean_inc(x_45); -lean_dec(x_4); -x_47 = lean_ctor_get(x_45, 0); -lean_inc(x_47); -x_48 = lean_ctor_get(x_45, 1); -lean_inc(x_48); -x_49 = lean_ctor_get(x_45, 2); -lean_inc(x_49); -if (lean_is_exclusive(x_45)) { - lean_ctor_release(x_45, 0); - lean_ctor_release(x_45, 1); - lean_ctor_release(x_45, 2); - x_50 = x_45; -} else { - lean_dec_ref(x_45); - x_50 = lean_box(0); -} -x_51 = lean_box(0); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_3); lean_inc(x_2); -lean_inc(x_1); -x_52 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___spec__1(x_1, x_2, x_3, x_49, x_51, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_52) == 0) { -lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; -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); -if (lean_is_scalar(x_50)) { - x_55 = lean_alloc_ctor(0, 3, 0); -} else { - x_55 = x_50; +lean_object* _tmp_2 = x_12; +lean_object* _tmp_3 = x_2; +lean_object* _tmp_8 = x_25; +x_3 = _tmp_2; +x_4 = _tmp_3; +x_9 = _tmp_8; } -lean_ctor_set(x_55, 0, x_47); -lean_ctor_set(x_55, 1, x_48); -lean_ctor_set(x_55, 2, x_53); -x_56 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_56, 0, x_55); -lean_ctor_set(x_56, 1, x_5); -x_4 = x_46; -x_5 = x_56; -x_12 = x_54; goto _start; } +} +} else { -lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; -lean_dec(x_50); -lean_dec(x_48); -lean_dec(x_47); -lean_dec(x_46); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); +uint8_t x_31; +lean_dec(x_12); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_58 = lean_ctor_get(x_52, 0); -lean_inc(x_58); -x_59 = lean_ctor_get(x_52, 1); -lean_inc(x_59); -if (lean_is_exclusive(x_52)) { - lean_ctor_release(x_52, 0); - lean_ctor_release(x_52, 1); - x_60 = x_52; -} else { - lean_dec_ref(x_52); - x_60 = lean_box(0); -} -if (lean_is_scalar(x_60)) { - x_61 = lean_alloc_ctor(1, 2, 0); -} else { - x_61 = x_60; -} -lean_ctor_set(x_61, 0, x_58); -lean_ctor_set(x_61, 1, x_59); -return x_61; -} +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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, 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; -x_14 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkIndFVar2Const(x_1, x_2, x_3); -x_15 = lean_box(0); -x_16 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___spec__2(x_4, x_5, x_14, x_6, x_15, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -return x_16; } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___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_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_5; -x_5 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___spec__1___lambda__1(x_1, x_2, x_3, x_4); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_5; -} -} -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___spec__1___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: +if (lean_obj_tag(x_3) == 0) { -lean_object* x_12; -x_12 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___spec__1___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_10); -lean_dec(x_9); +lean_object* x_10; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); -return x_12; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { -_start: -{ -lean_object* x_14; -x_14 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts(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_2); lean_dec(x_1); -return x_14; -} +x_10 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_10, 0, x_4); +lean_ctor_set(x_10, 1, x_9); +return x_10; } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1() { -_start: +else { -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_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1(uint8_t x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: +uint8_t x_11; +lean_dec(x_4); +x_11 = !lean_is_exclusive(x_3); +if (x_11 == 0) { -if (x_1 == 0) +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_12 = lean_ctor_get(x_3, 0); +x_13 = lean_ctor_get(x_3, 1); +x_14 = lean_ctor_get(x_12, 2); +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_n(x_2, 2); +lean_inc(x_1); +x_15 = l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__1(x_1, x_2, x_14, x_2, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_15) == 0) { -lean_object* x_12; lean_object* x_13; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -x_12 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_12); -lean_ctor_set(x_13, 1, x_11); -return x_13; -} -else +lean_object* x_16; lean_object* x_17; +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +lean_dec(x_16); +if (lean_obj_tag(x_17) == 0) { -if (x_2 == 0) +lean_object* x_18; +lean_free_object(x_3); +x_18 = lean_ctor_get(x_15, 1); +lean_inc(x_18); +lean_dec(x_15); +lean_inc(x_2); { -lean_object* x_14; lean_object* x_15; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -x_14 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; -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_object* _tmp_2 = x_13; +lean_object* _tmp_3 = x_2; +lean_object* _tmp_8 = x_18; +x_3 = _tmp_2; +x_4 = _tmp_3; +x_9 = _tmp_8; +} +goto _start; } else { -uint8_t x_16; lean_object* x_17; -x_16 = 0; -x_17 = l___private_Lean_Meta_Constructions_BRecOn_0__Lean_mkBelowOrIBelow(x_3, x_16, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_17) == 0) +uint8_t x_20; +lean_dec(x_13); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +lean_dec(x_1); +x_20 = !lean_is_exclusive(x_15); +if (x_20 == 0) { -uint8_t x_18; -x_18 = !lean_is_exclusive(x_17); -if (x_18 == 0) +lean_object* x_21; uint8_t x_22; +x_21 = lean_ctor_get(x_15, 0); +lean_dec(x_21); +x_22 = !lean_is_exclusive(x_17); +if (x_22 == 0) { -lean_object* x_19; lean_object* x_20; -x_19 = lean_ctor_get(x_17, 0); -lean_dec(x_19); -x_20 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; -lean_ctor_set(x_17, 0, x_20); -return x_17; +lean_object* x_23; +x_23 = lean_box(0); +lean_ctor_set_tag(x_3, 0); +lean_ctor_set(x_3, 1, x_23); +lean_ctor_set(x_3, 0, x_17); +lean_ctor_set(x_15, 0, x_3); +return x_15; } 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_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_22 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; -x_23 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_23, 0, x_22); -lean_ctor_set(x_23, 1, x_21); -return x_23; -} +x_25 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_25, 0, x_24); +x_26 = lean_box(0); +lean_ctor_set_tag(x_3, 0); +lean_ctor_set(x_3, 1, x_26); +lean_ctor_set(x_3, 0, x_25); +lean_ctor_set(x_15, 0, x_3); +return x_15; } -else -{ -uint8_t x_24; -x_24 = !lean_is_exclusive(x_17); -if (x_24 == 0) -{ -return x_17; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_17, 0); -x_26 = lean_ctor_get(x_17, 1); -lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_17); -x_27 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_26); -return x_27; -} +lean_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_15, 1); +lean_inc(x_27); +lean_dec(x_15); +x_28 = lean_ctor_get(x_17, 0); +lean_inc(x_28); +if (lean_is_exclusive(x_17)) { + lean_ctor_release(x_17, 0); + x_29 = x_17; +} else { + lean_dec_ref(x_17); + x_29 = lean_box(0); } +if (lean_is_scalar(x_29)) { + x_30 = lean_alloc_ctor(1, 1, 0); +} else { + x_30 = x_29; } +lean_ctor_set(x_30, 0, x_28); +x_31 = lean_box(0); +lean_ctor_set_tag(x_3, 0); +lean_ctor_set(x_3, 1, x_31); +lean_ctor_set(x_3, 0, x_30); +x_32 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_32, 0, x_3); +lean_ctor_set(x_32, 1, x_27); +return x_32; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__2(uint8_t x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: +else { -if (x_1 == 0) +uint8_t x_33; +lean_free_object(x_3); +lean_dec(x_13); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +lean_dec(x_1); +x_33 = !lean_is_exclusive(x_15); +if (x_33 == 0) { -lean_object* x_12; lean_object* x_13; -x_12 = lean_box(0); -x_13 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1(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; +return x_15; } else { -if (x_2 == 0) -{ -lean_object* x_14; lean_object* x_15; -x_14 = lean_box(0); -x_15 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1(x_1, x_2, x_3, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -return x_15; +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_15, 0); +x_35 = lean_ctor_get(x_15, 1); +lean_inc(x_35); +lean_inc(x_34); +lean_dec(x_15); +x_36 = lean_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_16; lean_object* x_17; -x_16 = 1; -lean_inc(x_10); -lean_inc(x_9); +lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_37 = lean_ctor_get(x_3, 0); +x_38 = lean_ctor_get(x_3, 1); +lean_inc(x_38); +lean_inc(x_37); +lean_dec(x_3); +x_39 = lean_ctor_get(x_37, 2); +lean_inc(x_39); +lean_dec(x_37); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_3); -x_17 = l___private_Lean_Meta_Constructions_BRecOn_0__Lean_mkBelowOrIBelow(x_3, x_16, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_17) == 0) +lean_inc(x_6); +lean_inc(x_5); +lean_inc_n(x_2, 2); +lean_inc(x_1); +x_40 = l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__1(x_1, x_2, x_39, x_2, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_40) == 0) { -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_17, 1); -lean_inc(x_19); -lean_dec(x_17); -x_20 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1(x_1, x_2, x_3, x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_19); -lean_dec(x_18); -return x_20; -} -else +lean_object* x_41; lean_object* x_42; +x_41 = lean_ctor_get(x_40, 0); +lean_inc(x_41); +x_42 = lean_ctor_get(x_41, 0); +lean_inc(x_42); +lean_dec(x_41); +if (lean_obj_tag(x_42) == 0) { -uint8_t x_21; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -x_21 = !lean_is_exclusive(x_17); -if (x_21 == 0) +lean_object* x_43; +x_43 = lean_ctor_get(x_40, 1); +lean_inc(x_43); +lean_dec(x_40); +lean_inc(x_2); { -return x_17; +lean_object* _tmp_2 = x_38; +lean_object* _tmp_3 = x_2; +lean_object* _tmp_8 = x_43; +x_3 = _tmp_2; +x_4 = _tmp_3; +x_9 = _tmp_8; +} +goto _start; } else { -lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_22 = lean_ctor_get(x_17, 0); -x_23 = lean_ctor_get(x_17, 1); -lean_inc(x_23); -lean_inc(x_22); -lean_dec(x_17); -x_24 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_24, 0, x_22); -lean_ctor_set(x_24, 1, x_23); -return x_24; -} +lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +lean_dec(x_38); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +lean_dec(x_1); +x_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_40); + x_46 = lean_box(0); } +x_47 = lean_ctor_get(x_42, 0); +lean_inc(x_47); +if (lean_is_exclusive(x_42)) { + lean_ctor_release(x_42, 0); + x_48 = x_42; +} else { + lean_dec_ref(x_42); + x_48 = lean_box(0); } +if (lean_is_scalar(x_48)) { + x_49 = lean_alloc_ctor(1, 1, 0); +} else { + x_49 = x_48; } +lean_ctor_set(x_49, 0, x_47); +x_50 = lean_box(0); +x_51 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_51, 0, x_49); +lean_ctor_set(x_51, 1, x_50); +if (lean_is_scalar(x_46)) { + x_52 = lean_alloc_ctor(0, 2, 0); +} else { + x_52 = x_46; } +lean_ctor_set(x_52, 0, x_51); +lean_ctor_set(x_52, 1, x_45); +return x_52; } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__3(uint8_t x_1, uint8_t 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) { -_start: -{ -if (x_1 == 0) -{ -lean_object* x_14; lean_object* x_15; -x_14 = lean_box(0); -x_15 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__2(x_1, x_2, x_3, x_14, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -return x_15; } else { -if (x_4 == 0) -{ -lean_object* x_16; lean_object* x_17; -x_16 = lean_box(0); -x_17 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__2(x_1, x_2, x_3, x_16, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -return x_17; -} -else -{ -if (x_5 == 0) -{ -lean_object* x_18; lean_object* x_19; -x_18 = lean_box(0); -x_19 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__2(x_1, x_2, x_3, x_18, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -return x_19; -} -else -{ -lean_object* x_20; -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_3); -x_20 = l_Lean_mkNoConfusion(x_3, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_20) == 0) -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_20, 1); -lean_inc(x_22); -lean_dec(x_20); -x_23 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__2(x_1, x_2, x_3, x_21, x_7, x_8, x_9, x_10, x_11, x_12, x_22); -lean_dec(x_21); -return x_23; -} -else -{ -uint8_t x_24; -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_3); -x_24 = !lean_is_exclusive(x_20); -if (x_24 == 0) -{ -return x_20; -} -else -{ -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_20, 0); -x_26 = lean_ctor_get(x_20, 1); -lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_20); -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_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; +lean_dec(x_38); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +lean_dec(x_1); +x_53 = lean_ctor_get(x_40, 0); +lean_inc(x_53); +x_54 = lean_ctor_get(x_40, 1); +lean_inc(x_54); +if (lean_is_exclusive(x_40)) { + lean_ctor_release(x_40, 0); + lean_ctor_release(x_40, 1); + x_55 = x_40; +} else { + lean_dec_ref(x_40); + x_55 = lean_box(0); } +if (lean_is_scalar(x_55)) { + x_56 = lean_alloc_ctor(1, 2, 0); +} else { + x_56 = x_55; } +lean_ctor_set(x_56, 0, x_53); +lean_ctor_set(x_56, 1, x_54); +return x_56; } } } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1(uint8_t x_1, uint8_t x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, size_t x_6, size_t x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +LEAN_EXPORT lean_object* l_List_foldl___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__3(lean_object* x_1, lean_object* x_2) { _start: { -uint8_t x_16; -x_16 = lean_usize_dec_lt(x_7, x_6); -if (x_16 == 0) +if (lean_obj_tag(x_2) == 0) { -lean_object* x_17; -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_8); -lean_ctor_set(x_17, 1, x_15); -return x_17; +return x_1; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; -lean_dec(x_8); -x_18 = lean_array_uget(x_5, x_7); -x_19 = lean_ctor_get(x_18, 4); -lean_inc(x_19); -lean_dec(x_18); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_19); -x_20 = l_mkRecOn(x_19, x_11, x_12, x_13, x_14, x_15); -if (lean_obj_tag(x_20) == 0) -{ -if (x_3 == 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_box(0); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -x_23 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__3(x_3, x_4, x_19, x_1, x_2, x_22, x_9, x_10, x_11, x_12, x_13, x_14, x_21); -if (lean_obj_tag(x_23) == 0) -{ -lean_object* x_24; -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -if (lean_obj_tag(x_24) == 0) -{ -uint8_t x_25; -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -x_25 = !lean_is_exclusive(x_23); -if (x_25 == 0) +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; +x_3 = lean_ctor_get(x_2, 0); +x_4 = lean_ctor_get(x_2, 1); +x_5 = lean_ctor_get(x_3, 2); +x_6 = lean_unsigned_to_nat(0u); +x_7 = l_List_lengthTRAux___rarg(x_5, x_6); +x_8 = lean_nat_dec_le(x_1, x_7); +if (x_8 == 0) { -lean_object* x_26; lean_object* x_27; -x_26 = lean_ctor_get(x_23, 0); -lean_dec(x_26); -x_27 = lean_ctor_get(x_24, 0); -lean_inc(x_27); -lean_dec(x_24); -lean_ctor_set(x_23, 0, x_27); -return x_23; +lean_dec(x_7); +x_2 = x_4; +goto _start; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_28 = lean_ctor_get(x_23, 1); -lean_inc(x_28); -lean_dec(x_23); -x_29 = lean_ctor_get(x_24, 0); -lean_inc(x_29); -lean_dec(x_24); -x_30 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_30, 0, x_29); -lean_ctor_set(x_30, 1, x_28); -return x_30; +lean_dec(x_1); +x_1 = x_7; +x_2 = x_4; +goto _start; } } -else -{ -lean_object* x_31; lean_object* x_32; size_t x_33; size_t x_34; -x_31 = lean_ctor_get(x_23, 1); -lean_inc(x_31); -lean_dec(x_23); -x_32 = lean_ctor_get(x_24, 0); -lean_inc(x_32); -lean_dec(x_24); -x_33 = 1; -x_34 = lean_usize_add(x_7, x_33); -x_7 = x_34; -x_8 = x_32; -x_15 = x_31; -goto _start; } } -else -{ -uint8_t x_36; -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -x_36 = !lean_is_exclusive(x_23); -if (x_36 == 0) +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___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: { -return x_23; +uint8_t x_7; lean_object* x_8; lean_object* x_9; +x_7 = 0; +x_8 = lean_box(x_7); +x_9 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_9, 0, x_8); +lean_ctor_set(x_9, 1, x_6); +return x_9; } -else -{ -lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_37 = lean_ctor_get(x_23, 0); -x_38 = lean_ctor_get(x_23, 1); -lean_inc(x_38); -lean_inc(x_37); -lean_dec(x_23); -x_39 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_39, 0, x_37); -lean_ctor_set(x_39, 1, x_38); -return x_39; } +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___lambda__2___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___lambda__1___boxed), 6, 0); +return x_1; } } -else +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: { -lean_object* x_40; lean_object* x_41; -x_40 = lean_ctor_get(x_20, 1); -lean_inc(x_40); -lean_dec(x_20); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_19); -x_41 = l_Lean_mkCasesOn(x_19, x_11, x_12, x_13, x_14, x_40); -if (lean_obj_tag(x_41) == 0) +lean_object* x_9; lean_object* x_10; +x_9 = l_Lean_Elab_Command_withCtorRef___rarg___closed__1; +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_10 = l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__2(x_1, x_9, x_2, x_9, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_10) == 0) { -lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_ctor_get(x_41, 0); -lean_inc(x_42); -x_43 = lean_ctor_get(x_41, 1); -lean_inc(x_43); -lean_dec(x_41); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); +lean_object* x_11; lean_object* x_12; +x_11 = lean_ctor_get(x_10, 0); lean_inc(x_11); -x_44 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__3(x_3, x_4, x_19, x_1, x_2, x_42, x_9, x_10, x_11, x_12, x_13, x_14, x_43); -lean_dec(x_42); -if (lean_obj_tag(x_44) == 0) -{ -lean_object* x_45; -x_45 = lean_ctor_get(x_44, 0); -lean_inc(x_45); -if (lean_obj_tag(x_45) == 0) -{ -uint8_t x_46; -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); lean_dec(x_11); -x_46 = !lean_is_exclusive(x_44); -if (x_46 == 0) -{ -lean_object* x_47; lean_object* x_48; -x_47 = lean_ctor_get(x_44, 0); -lean_dec(x_47); -x_48 = lean_ctor_get(x_45, 0); -lean_inc(x_48); -lean_dec(x_45); -lean_ctor_set(x_44, 0, x_48); -return x_44; -} -else +if (lean_obj_tag(x_12) == 0) { -lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_49 = lean_ctor_get(x_44, 1); -lean_inc(x_49); -lean_dec(x_44); -x_50 = lean_ctor_get(x_45, 0); -lean_inc(x_50); -lean_dec(x_45); -x_51 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_51, 0, x_50); -lean_ctor_set(x_51, 1, x_49); -return x_51; -} +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_13 = lean_ctor_get(x_10, 1); +lean_inc(x_13); +lean_dec(x_10); +x_14 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___lambda__2___closed__1; +x_15 = lean_box(0); +x_16 = lean_apply_6(x_14, x_15, x_4, x_5, x_6, x_7, x_13); +return x_16; } else { -lean_object* x_52; lean_object* x_53; size_t x_54; size_t x_55; -x_52 = lean_ctor_get(x_44, 1); -lean_inc(x_52); -lean_dec(x_44); -x_53 = lean_ctor_get(x_45, 0); -lean_inc(x_53); -lean_dec(x_45); -x_54 = 1; -x_55 = lean_usize_add(x_7, x_54); -x_7 = x_55; -x_8 = x_53; -x_15 = x_52; -goto _start; -} -} -else +uint8_t x_17; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_17 = !lean_is_exclusive(x_10); +if (x_17 == 0) { -uint8_t x_57; -lean_dec(x_14); -lean_dec(x_13); +lean_object* x_18; lean_object* x_19; +x_18 = lean_ctor_get(x_10, 0); +lean_dec(x_18); +x_19 = lean_ctor_get(x_12, 0); +lean_inc(x_19); lean_dec(x_12); -lean_dec(x_11); -x_57 = !lean_is_exclusive(x_44); -if (x_57 == 0) -{ -return x_44; +lean_ctor_set(x_10, 0, x_19); +return x_10; } else { -lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_58 = lean_ctor_get(x_44, 0); -x_59 = lean_ctor_get(x_44, 1); -lean_inc(x_59); -lean_inc(x_58); -lean_dec(x_44); -x_60 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_60, 0, x_58); -lean_ctor_set(x_60, 1, x_59); -return x_60; +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_10, 1); +lean_inc(x_20); +lean_dec(x_10); +x_21 = lean_ctor_get(x_12, 0); +lean_inc(x_21); +lean_dec(x_12); +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 { -uint8_t x_61; -lean_dec(x_19); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -x_61 = !lean_is_exclusive(x_41); -if (x_61 == 0) +uint8_t x_23; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_23 = !lean_is_exclusive(x_10); +if (x_23 == 0) { -return x_41; +return x_10; } else { -lean_object* x_62; lean_object* x_63; lean_object* x_64; -x_62 = lean_ctor_get(x_41, 0); -x_63 = lean_ctor_get(x_41, 1); -lean_inc(x_63); -lean_inc(x_62); -lean_dec(x_41); -x_64 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_64, 0, x_62); -lean_ctor_set(x_64, 1, x_63); -return x_64; +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_10, 0); +x_25 = lean_ctor_get(x_10, 1); +lean_inc(x_25); +lean_inc(x_24); +lean_dec(x_10); +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_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate(lean_object* x_1, 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_65; -lean_dec(x_19); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -x_65 = !lean_is_exclusive(x_20); -if (x_65 == 0) +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_List_foldl___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__3(x_8, x_2); +x_10 = lean_unsigned_to_nat(1u); +x_11 = lean_nat_dec_eq(x_9, x_10); +lean_dec(x_9); +if (x_11 == 0) { -return x_20; +uint8_t x_12; lean_object* x_13; lean_object* 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_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_7); +return x_14; } else { -lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_66 = lean_ctor_get(x_20, 0); -x_67 = lean_ctor_get(x_20, 1); -lean_inc(x_67); -lean_inc(x_66); -lean_dec(x_20); -x_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_15; lean_object* x_16; +x_15 = lean_box(0); +x_16 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___lambda__2(x_1, x_2, x_15, x_3, x_4, x_5, x_6, x_7); +return x_16; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__2___lambda__1(uint8_t x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -if (x_1 == 0) -{ -lean_object* x_12; lean_object* x_13; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); +lean_object* x_9; +x_9 = l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); -x_12 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_12); -lean_ctor_set(x_13, 1, x_11); -return x_13; +lean_dec(x_2); +lean_dec(x_1); +return x_9; } -else +} +LEAN_EXPORT lean_object* l_List_foldl___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__3___boxed(lean_object* x_1, lean_object* x_2) { +_start: { -if (x_2 == 0) +lean_object* x_3; +x_3 = l_List_foldl___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___spec__3(x_1, x_2); +lean_dec(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___lambda__1___boxed(lean_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_14; lean_object* x_15; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); +lean_object* x_7; +x_7 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___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); -x_14 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; -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_dec(x_2); +lean_dec(x_1); +return x_7; } -else +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___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_16; lean_object* x_17; -x_16 = 1; -x_17 = l_Lean_mkBRecOnOrBInductionOn(x_3, x_16, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_17) == 0) +lean_object* x_9; +x_9 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_3); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_assignLevelMVar___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: { -uint8_t x_18; -x_18 = !lean_is_exclusive(x_17); -if (x_18 == 0) +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_10 = lean_st_ref_take(x_6, x_9); +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_10, 1); +lean_inc(x_13); +lean_dec(x_10); +x_14 = !lean_is_exclusive(x_11); +if (x_14 == 0) { -lean_object* x_19; lean_object* x_20; -x_19 = lean_ctor_get(x_17, 0); -lean_dec(x_19); -x_20 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; -lean_ctor_set(x_17, 0, x_20); -return x_17; +lean_object* x_15; uint8_t x_16; +x_15 = lean_ctor_get(x_11, 0); +lean_dec(x_15); +x_16 = !lean_is_exclusive(x_12); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; +x_17 = lean_ctor_get(x_12, 6); +x_18 = l_Lean_PersistentHashMap_insert___at_Lean_assignLevelMVar___spec__1(x_17, x_1, x_2); +lean_ctor_set(x_12, 6, x_18); +x_19 = lean_st_ref_set(x_6, x_11, 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_box(0); +lean_ctor_set(x_19, 0, x_22); +return x_19; } else { -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_17, 1); -lean_inc(x_21); -lean_dec(x_17); -x_22 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; -x_23 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_23, 0, x_22); -lean_ctor_set(x_23, 1, x_21); -return x_23; +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_19, 1); +lean_inc(x_23); +lean_dec(x_19); +x_24 = lean_box(0); +x_25 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_25, 0, x_24); +lean_ctor_set(x_25, 1, x_23); +return x_25; } } else { -uint8_t x_24; -x_24 = !lean_is_exclusive(x_17); -if (x_24 == 0) -{ -return x_17; +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; +x_26 = lean_ctor_get(x_12, 0); +x_27 = lean_ctor_get(x_12, 1); +x_28 = lean_ctor_get(x_12, 2); +x_29 = lean_ctor_get(x_12, 3); +x_30 = lean_ctor_get(x_12, 4); +x_31 = lean_ctor_get(x_12, 5); +x_32 = lean_ctor_get(x_12, 6); +x_33 = lean_ctor_get(x_12, 7); +x_34 = lean_ctor_get(x_12, 8); +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_dec(x_12); +x_35 = l_Lean_PersistentHashMap_insert___at_Lean_assignLevelMVar___spec__1(x_32, x_1, x_2); +x_36 = lean_alloc_ctor(0, 9, 0); +lean_ctor_set(x_36, 0, x_26); +lean_ctor_set(x_36, 1, x_27); +lean_ctor_set(x_36, 2, x_28); +lean_ctor_set(x_36, 3, x_29); +lean_ctor_set(x_36, 4, x_30); +lean_ctor_set(x_36, 5, x_31); +lean_ctor_set(x_36, 6, x_35); +lean_ctor_set(x_36, 7, x_33); +lean_ctor_set(x_36, 8, x_34); +lean_ctor_set(x_11, 0, x_36); +x_37 = lean_st_ref_set(x_6, x_11, x_13); +x_38 = lean_ctor_get(x_37, 1); +lean_inc(x_38); +if (lean_is_exclusive(x_37)) { + lean_ctor_release(x_37, 0); + lean_ctor_release(x_37, 1); + x_39 = x_37; +} else { + lean_dec_ref(x_37); + x_39 = lean_box(0); +} +x_40 = lean_box(0); +if (lean_is_scalar(x_39)) { + x_41 = lean_alloc_ctor(0, 2, 0); +} else { + x_41 = x_39; +} +lean_ctor_set(x_41, 0, x_40); +lean_ctor_set(x_41, 1, x_38); +return x_41; +} } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_17, 0); -x_26 = lean_ctor_get(x_17, 1); -lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_17); -x_27 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_26); -return x_27; +lean_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_42 = lean_ctor_get(x_11, 1); +x_43 = lean_ctor_get(x_11, 2); +x_44 = lean_ctor_get(x_11, 3); +x_45 = lean_ctor_get(x_11, 4); +lean_inc(x_45); +lean_inc(x_44); +lean_inc(x_43); +lean_inc(x_42); +lean_dec(x_11); +x_46 = lean_ctor_get(x_12, 0); +lean_inc(x_46); +x_47 = lean_ctor_get(x_12, 1); +lean_inc(x_47); +x_48 = lean_ctor_get(x_12, 2); +lean_inc(x_48); +x_49 = lean_ctor_get(x_12, 3); +lean_inc(x_49); +x_50 = lean_ctor_get(x_12, 4); +lean_inc(x_50); +x_51 = lean_ctor_get(x_12, 5); +lean_inc(x_51); +x_52 = lean_ctor_get(x_12, 6); +lean_inc(x_52); +x_53 = lean_ctor_get(x_12, 7); +lean_inc(x_53); +x_54 = lean_ctor_get(x_12, 8); +lean_inc(x_54); +if (lean_is_exclusive(x_12)) { + lean_ctor_release(x_12, 0); + lean_ctor_release(x_12, 1); + lean_ctor_release(x_12, 2); + lean_ctor_release(x_12, 3); + lean_ctor_release(x_12, 4); + lean_ctor_release(x_12, 5); + lean_ctor_release(x_12, 6); + lean_ctor_release(x_12, 7); + lean_ctor_release(x_12, 8); + x_55 = x_12; +} else { + lean_dec_ref(x_12); + x_55 = lean_box(0); +} +x_56 = l_Lean_PersistentHashMap_insert___at_Lean_assignLevelMVar___spec__1(x_52, x_1, x_2); +if (lean_is_scalar(x_55)) { + x_57 = lean_alloc_ctor(0, 9, 0); +} else { + x_57 = x_55; } +lean_ctor_set(x_57, 0, x_46); +lean_ctor_set(x_57, 1, x_47); +lean_ctor_set(x_57, 2, x_48); +lean_ctor_set(x_57, 3, x_49); +lean_ctor_set(x_57, 4, x_50); +lean_ctor_set(x_57, 5, x_51); +lean_ctor_set(x_57, 6, x_56); +lean_ctor_set(x_57, 7, x_53); +lean_ctor_set(x_57, 8, x_54); +x_58 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_58, 0, x_57); +lean_ctor_set(x_58, 1, x_42); +lean_ctor_set(x_58, 2, x_43); +lean_ctor_set(x_58, 3, x_44); +lean_ctor_set(x_58, 4, x_45); +x_59 = lean_st_ref_set(x_6, x_58, x_13); +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; +} else { + lean_dec_ref(x_59); + x_61 = lean_box(0); } +x_62 = lean_box(0); +if (lean_is_scalar(x_61)) { + x_63 = lean_alloc_ctor(0, 2, 0); +} else { + x_63 = x_61; } +lean_ctor_set(x_63, 0, x_62); +lean_ctor_set(x_63, 1, x_60); +return x_63; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__2(uint8_t x_1, uint8_t 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_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -uint8_t x_14; -x_14 = lean_usize_dec_lt(x_5, x_4); -if (x_14 == 0) +if (lean_obj_tag(x_1) == 0) { -lean_object* x_15; -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -x_15 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_15, 0, x_6); -lean_ctor_set(x_15, 1, x_13); -return x_15; +lean_object* x_10; lean_object* x_11; +x_10 = l_List_reverse___rarg(x_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); +return x_11; } else { -lean_object* x_16; -lean_dec(x_6); -x_16 = lean_array_uget(x_3, x_5); -if (x_1 == 0) -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_16, 4); -lean_inc(x_17); -lean_dec(x_16); -x_18 = lean_box(0); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -x_19 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__2___lambda__1(x_1, x_2, x_17, x_18, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_19) == 0) +uint8_t x_12; +x_12 = !lean_is_exclusive(x_1); +if (x_12 == 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_13; uint8_t x_14; +x_13 = lean_ctor_get(x_1, 0); +x_14 = !lean_is_exclusive(x_13); +if (x_14 == 0) { -uint8_t x_21; -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -x_21 = !lean_is_exclusive(x_19); -if (x_21 == 0) +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_15 = lean_ctor_get(x_1, 1); +x_16 = lean_ctor_get(x_13, 1); +x_17 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_16, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); +lean_dec(x_17); +lean_ctor_set(x_13, 1, x_18); +lean_ctor_set(x_1, 1, x_2); { -lean_object* x_22; lean_object* x_23; -x_22 = lean_ctor_get(x_19, 0); -lean_dec(x_22); -x_23 = lean_ctor_get(x_20, 0); -lean_inc(x_23); -lean_dec(x_20); -lean_ctor_set(x_19, 0, x_23); -return x_19; +lean_object* _tmp_0 = x_15; +lean_object* _tmp_1 = x_1; +lean_object* _tmp_8 = x_19; +x_1 = _tmp_0; +x_2 = _tmp_1; +x_9 = _tmp_8; +} +goto _start; } else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_19, 1); -lean_inc(x_24); -lean_dec(x_19); -x_25 = lean_ctor_get(x_20, 0); +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_21 = lean_ctor_get(x_1, 1); +x_22 = lean_ctor_get(x_13, 0); +x_23 = lean_ctor_get(x_13, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_13); +x_24 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_23, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_25 = lean_ctor_get(x_24, 0); lean_inc(x_25); -lean_dec(x_20); -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 +x_26 = lean_ctor_get(x_24, 1); +lean_inc(x_26); +lean_dec(x_24); +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_22); +lean_ctor_set(x_27, 1, x_25); +lean_ctor_set(x_1, 1, x_2); +lean_ctor_set(x_1, 0, x_27); { -lean_object* x_27; lean_object* x_28; size_t x_29; size_t x_30; -x_27 = lean_ctor_get(x_19, 1); -lean_inc(x_27); -lean_dec(x_19); -x_28 = lean_ctor_get(x_20, 0); -lean_inc(x_28); -lean_dec(x_20); -x_29 = 1; -x_30 = lean_usize_add(x_5, x_29); -x_5 = x_30; -x_6 = x_28; -x_13 = x_27; +lean_object* _tmp_0 = x_21; +lean_object* _tmp_1 = x_1; +lean_object* _tmp_8 = x_26; +x_1 = _tmp_0; +x_2 = _tmp_1; +x_9 = _tmp_8; +} goto _start; } } else { -uint8_t x_32; -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -x_32 = !lean_is_exclusive(x_19); -if (x_32 == 0) -{ -return x_19; +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_29 = lean_ctor_get(x_1, 0); +x_30 = lean_ctor_get(x_1, 1); +lean_inc(x_30); +lean_inc(x_29); +lean_dec(x_1); +x_31 = lean_ctor_get(x_29, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_29, 1); +lean_inc(x_32); +if (lean_is_exclusive(x_29)) { + lean_ctor_release(x_29, 0); + lean_ctor_release(x_29, 1); + x_33 = x_29; +} else { + lean_dec_ref(x_29); + x_33 = lean_box(0); } -else -{ -lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_33 = lean_ctor_get(x_19, 0); -x_34 = lean_ctor_get(x_19, 1); -lean_inc(x_34); -lean_inc(x_33); -lean_dec(x_19); -x_35 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_35, 0, x_33); -lean_ctor_set(x_35, 1, x_34); -return x_35; +x_34 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_32, 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); +if (lean_is_scalar(x_33)) { + x_37 = lean_alloc_ctor(0, 2, 0); +} else { + x_37 = x_33; +} +lean_ctor_set(x_37, 0, x_31); +lean_ctor_set(x_37, 1, x_35); +x_38 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_38, 0, x_37); +lean_ctor_set(x_38, 1, x_2); +x_1 = x_30; +x_2 = x_38; +x_9 = x_36; +goto _start; } } } -else +} +LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: { -if (x_2 == 0) +if (lean_obj_tag(x_1) == 0) { -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_16, 4); -lean_inc(x_36); -lean_dec(x_16); -x_37 = lean_box(0); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -x_38 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__2___lambda__1(x_1, x_2, x_36, x_37, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_38) == 0) +lean_object* x_10; lean_object* x_11; +x_10 = l_List_reverse___rarg(x_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); +return x_11; +} +else { -lean_object* x_39; -x_39 = lean_ctor_get(x_38, 0); -lean_inc(x_39); -if (lean_obj_tag(x_39) == 0) +uint8_t x_12; +x_12 = !lean_is_exclusive(x_1); +if (x_12 == 0) { -uint8_t x_40; -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -x_40 = !lean_is_exclusive(x_38); -if (x_40 == 0) +lean_object* x_13; uint8_t x_14; +x_13 = lean_ctor_get(x_1, 0); +x_14 = !lean_is_exclusive(x_13); +if (x_14 == 0) { -lean_object* x_41; lean_object* x_42; -x_41 = lean_ctor_get(x_38, 0); -lean_dec(x_41); -x_42 = lean_ctor_get(x_39, 0); -lean_inc(x_42); -lean_dec(x_39); -lean_ctor_set(x_38, 0, x_42); -return x_38; -} -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; +x_15 = lean_ctor_get(x_1, 1); +x_16 = lean_ctor_get(x_13, 1); +x_17 = lean_ctor_get(x_13, 2); +x_18 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_16, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +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_box(0); +x_22 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___spec__2(x_17, x_21, x_3, x_4, x_5, x_6, x_7, x_8, 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_ctor_set(x_13, 2, x_23); +lean_ctor_set(x_13, 1, x_19); +lean_ctor_set(x_1, 1, x_2); { -lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_43 = lean_ctor_get(x_38, 1); -lean_inc(x_43); -lean_dec(x_38); -x_44 = lean_ctor_get(x_39, 0); -lean_inc(x_44); -lean_dec(x_39); -x_45 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_45, 0, x_44); -lean_ctor_set(x_45, 1, x_43); -return x_45; -} +lean_object* _tmp_0 = x_15; +lean_object* _tmp_1 = x_1; +lean_object* _tmp_8 = x_24; +x_1 = _tmp_0; +x_2 = _tmp_1; +x_9 = _tmp_8; } -else -{ -lean_object* x_46; lean_object* x_47; size_t x_48; size_t x_49; -x_46 = lean_ctor_get(x_38, 1); -lean_inc(x_46); -lean_dec(x_38); -x_47 = lean_ctor_get(x_39, 0); -lean_inc(x_47); -lean_dec(x_39); -x_48 = 1; -x_49 = lean_usize_add(x_5, x_48); -x_5 = x_49; -x_6 = x_47; -x_13 = x_46; goto _start; } -} else { -uint8_t x_51; -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -x_51 = !lean_is_exclusive(x_38); -if (x_51 == 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; +x_26 = lean_ctor_get(x_1, 1); +x_27 = lean_ctor_get(x_13, 0); +x_28 = lean_ctor_get(x_13, 1); +x_29 = lean_ctor_get(x_13, 2); +lean_inc(x_29); +lean_inc(x_28); +lean_inc(x_27); +lean_dec(x_13); +x_30 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_28, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +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_box(0); +x_34 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___spec__2(x_29, x_33, x_3, x_4, x_5, x_6, x_7, x_8, 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_alloc_ctor(0, 3, 0); +lean_ctor_set(x_37, 0, x_27); +lean_ctor_set(x_37, 1, x_31); +lean_ctor_set(x_37, 2, x_35); +lean_ctor_set(x_1, 1, x_2); +lean_ctor_set(x_1, 0, x_37); { -return x_38; +lean_object* _tmp_0 = x_26; +lean_object* _tmp_1 = x_1; +lean_object* _tmp_8 = x_36; +x_1 = _tmp_0; +x_2 = _tmp_1; +x_9 = _tmp_8; +} +goto _start; +} } else { -lean_object* x_52; lean_object* x_53; lean_object* x_54; -x_52 = lean_ctor_get(x_38, 0); -x_53 = lean_ctor_get(x_38, 1); -lean_inc(x_53); -lean_inc(x_52); -lean_dec(x_38); -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_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_39 = lean_ctor_get(x_1, 0); +x_40 = lean_ctor_get(x_1, 1); +lean_inc(x_40); +lean_inc(x_39); +lean_dec(x_1); +x_41 = lean_ctor_get(x_39, 0); +lean_inc(x_41); +x_42 = lean_ctor_get(x_39, 1); +lean_inc(x_42); +x_43 = lean_ctor_get(x_39, 2); +lean_inc(x_43); +if (lean_is_exclusive(x_39)) { + lean_ctor_release(x_39, 0); + lean_ctor_release(x_39, 1); + lean_ctor_release(x_39, 2); + x_44 = x_39; +} else { + lean_dec_ref(x_39); + x_44 = lean_box(0); +} +x_45 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_42, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_46 = lean_ctor_get(x_45, 0); +lean_inc(x_46); +x_47 = lean_ctor_get(x_45, 1); +lean_inc(x_47); +lean_dec(x_45); +x_48 = lean_box(0); +x_49 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___spec__2(x_43, x_48, x_3, x_4, x_5, x_6, x_7, x_8, x_47); +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); +if (lean_is_scalar(x_44)) { + x_52 = lean_alloc_ctor(0, 3, 0); +} else { + x_52 = x_44; +} +lean_ctor_set(x_52, 0, x_41); +lean_ctor_set(x_52, 1, x_46); +lean_ctor_set(x_52, 2, x_50); +x_53 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_53, 0, x_52); +lean_ctor_set(x_53, 1, x_2); +x_1 = x_40; +x_2 = x_53; +x_9 = x_51; +goto _start; } } } -else -{ -lean_object* x_55; uint8_t x_56; lean_object* x_57; -x_55 = lean_ctor_get(x_16, 4); -lean_inc(x_55); -lean_dec(x_16); -x_56 = 0; -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_55); -x_57 = l_Lean_mkBRecOnOrBInductionOn(x_55, x_56, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_57) == 0) +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___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_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_object* x_14; lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -x_60 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__2___lambda__1(x_1, x_2, x_55, x_58, x_7, x_8, x_9, x_10, x_11, x_12, x_59); -lean_dec(x_58); -if (lean_obj_tag(x_60) == 0) -{ -lean_object* x_61; -x_61 = lean_ctor_get(x_60, 0); -lean_inc(x_61); -if (lean_obj_tag(x_61) == 0) -{ -uint8_t x_62; -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -x_62 = !lean_is_exclusive(x_60); -if (x_62 == 0) -{ -lean_object* x_63; lean_object* x_64; -x_63 = lean_ctor_get(x_60, 0); -lean_dec(x_63); -x_64 = lean_ctor_get(x_61, 0); -lean_inc(x_64); -lean_dec(x_61); -lean_ctor_set(x_60, 0, x_64); -return x_60; -} -else -{ -lean_object* x_65; lean_object* x_66; lean_object* x_67; -x_65 = lean_ctor_get(x_60, 1); -lean_inc(x_65); -lean_dec(x_60); -x_66 = lean_ctor_get(x_61, 0); -lean_inc(x_66); -lean_dec(x_61); -x_67 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_67, 0, x_66); -lean_ctor_set(x_67, 1, x_65); -return x_67; -} -} -else -{ -lean_object* x_68; lean_object* x_69; size_t x_70; size_t x_71; -x_68 = lean_ctor_get(x_60, 1); -lean_inc(x_68); -lean_dec(x_60); -x_69 = lean_ctor_get(x_61, 0); -lean_inc(x_69); -lean_dec(x_61); -x_70 = 1; -x_71 = lean_usize_add(x_5, x_70); -x_5 = x_71; -x_6 = x_69; -x_13 = x_68; -goto _start; -} -} -else +lean_inc(x_2); +x_14 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isPropCandidate(x_1, x_2, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_14) == 0) { -uint8_t x_73; +lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +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_Lean_Elab_Command_mkResultUniverse(x_3, x_4, x_17); +x_19 = l_Lean_Level_mvarId_x21(x_5); +x_20 = l_Lean_assignLevelMVar___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___spec__1(x_19, x_18, x_7, x_8, x_9, x_10, x_11, x_12, x_16); +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +x_22 = lean_box(0); +x_23 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___spec__3(x_2, x_22, x_7, x_8, x_9, x_10, x_11, x_12, x_21); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -x_73 = !lean_is_exclusive(x_60); -if (x_73 == 0) -{ -return x_60; -} -else -{ -lean_object* x_74; lean_object* x_75; lean_object* x_76; -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); -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; -} -} +return x_23; } else { -uint8_t x_77; -lean_dec(x_55); +uint8_t x_24; lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -x_77 = !lean_is_exclusive(x_57); -if (x_77 == 0) +lean_dec(x_3); +lean_dec(x_2); +x_24 = !lean_is_exclusive(x_14); +if (x_24 == 0) { -return x_57; +return x_14; } else { -lean_object* x_78; lean_object* x_79; lean_object* x_80; -x_78 = lean_ctor_get(x_57, 0); -x_79 = lean_ctor_get(x_57, 1); -lean_inc(x_79); -lean_inc(x_78); -lean_dec(x_57); -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; -} -} -} -} -} -} -} -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Eq", 2, 2); -return x_1; +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_14, 0); +x_26 = lean_ctor_get(x_14, 1); +lean_inc(x_26); +lean_inc(x_25); +lean_dec(x_14); +x_27 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +return x_27; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___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_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__3() { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("HEq", 3, 3); +x_1 = lean_mk_string_unchecked("updateResultingUniverse us: ", 28, 28); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__4() { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___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_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__3; -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_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__5() { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__3() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("PUnit", 5, 5); +x_1 = lean_mk_string_unchecked(", r: ", 5, 5); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__6() { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___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_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__5; -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_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__7() { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__5() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("Prod", 4, 4); +x_1 = lean_mk_string_unchecked(", rOffset: ", 11, 11); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__8() { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___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_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__7; -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_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__5; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions(lean_object* x_1, lean_object* x_2, lean_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_Inductive_0__Lean_Elab_Command_updateResultingUniverse___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_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; lean_object* x_17; uint8_t x_18; lean_object* x_19; uint8_t x_20; size_t x_21; size_t x_22; lean_object* x_23; lean_object* x_24; -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, 0); -lean_inc(x_12); -lean_dec(x_10); -x_13 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__2; -lean_inc(x_12); -x_14 = l_Lean_Environment_contains(x_12, x_13); -x_15 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__4; -lean_inc(x_12); -x_16 = l_Lean_Environment_contains(x_12, x_15); -x_17 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__6; +lean_object* x_14; lean_inc(x_12); -x_18 = l_Lean_Environment_contains(x_12, x_17); -x_19 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__8; -x_20 = l_Lean_Environment_contains(x_12, x_19); -x_21 = lean_array_size(x_1); -x_22 = 0; -x_23 = lean_box(0); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -x_24 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1(x_14, x_16, x_18, x_20, x_1, x_21, x_22, x_23, x_2, x_3, x_4, x_5, x_6, x_7, x_11); -if (lean_obj_tag(x_24) == 0) -{ -lean_object* x_25; lean_object* x_26; -x_25 = lean_ctor_get(x_24, 1); -lean_inc(x_25); -lean_dec(x_24); -x_26 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__2(x_18, x_20, x_1, x_21, x_22, x_23, x_2, x_3, x_4, x_5, x_6, x_7, 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_inc(x_3); +lean_inc(x_2); +x_14 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses(x_1, x_2, x_3, x_4, x_5, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_14) == 0) { -lean_object* x_28; -x_28 = lean_ctor_get(x_26, 0); -lean_dec(x_28); -lean_ctor_set(x_26, 0, x_23); -return x_26; -} -else +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; +x_15 = lean_ctor_get(x_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_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__3; +x_18 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_17, x_7, x_8, x_9, x_10, x_11, x_12, x_16); +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +x_20 = lean_unbox(x_19); +lean_dec(x_19); +if (x_20 == 0) { -lean_object* x_29; lean_object* x_30; -x_29 = lean_ctor_get(x_26, 1); -lean_inc(x_29); -lean_dec(x_26); -x_30 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_30, 0, x_23); -lean_ctor_set(x_30, 1, x_29); -return x_30; -} +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_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__1(x_4, x_5, x_15, x_3, x_2, x_22, x_7, x_8, x_9, x_10, x_11, x_12, x_21); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_2); +lean_dec(x_3); +return x_23; } else { -uint8_t x_31; -x_31 = !lean_is_exclusive(x_26); -if (x_31 == 0) -{ -return x_26; -} -else +uint8_t x_24; +x_24 = !lean_is_exclusive(x_18); +if (x_24 == 0) { -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_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; +x_25 = lean_ctor_get(x_18, 1); +x_26 = lean_ctor_get(x_18, 0); 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; -} -} -} -else -{ -uint8_t x_35; +lean_inc(x_15); +x_27 = lean_array_to_list(x_15); +x_28 = lean_box(0); +x_29 = l_List_mapTR_loop___at_Lean_Meta_Match_mkMatcher___spec__6(x_27, x_28); +x_30 = l_Lean_MessageData_ofList(x_29); +x_31 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__2; +lean_ctor_set_tag(x_18, 7); +lean_ctor_set(x_18, 1, x_30); +lean_ctor_set(x_18, 0, x_31); +x_32 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__4; +x_33 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_33, 0, x_18); +lean_ctor_set(x_33, 1, x_32); +lean_inc(x_2); +x_34 = l_Lean_MessageData_ofLevel(x_2); +x_35 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +x_36 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__6; +x_37 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +lean_inc(x_3); +x_38 = l___private_Init_Data_Repr_0__Nat_reprFast(x_3); +x_39 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_39, 0, x_38); +x_40 = l_Lean_MessageData_ofFormat(x_39); +x_41 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_41, 0, x_37); +lean_ctor_set(x_41, 1, x_40); +x_42 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +x_43 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_43, 0, x_41); +lean_ctor_set(x_43, 1, x_42); +x_44 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_17, x_43, x_7, x_8, x_9, x_10, x_11, x_12, x_25); +x_45 = lean_ctor_get(x_44, 0); +lean_inc(x_45); +x_46 = lean_ctor_get(x_44, 1); +lean_inc(x_46); +lean_dec(x_44); +x_47 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__1(x_4, x_5, x_15, x_3, x_2, x_45, x_7, x_8, x_9, x_10, x_11, x_12, x_46); +lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -x_35 = !lean_is_exclusive(x_24); -if (x_35 == 0) -{ -return x_24; +lean_dec(x_45); +lean_dec(x_2); +lean_dec(x_3); +return x_47; } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_24, 0); -x_37 = lean_ctor_get(x_24, 1); -lean_inc(x_37); -lean_inc(x_36); -lean_dec(x_24); -x_38 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -return x_38; -} -} -} -} -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -uint8_t x_12; uint8_t x_13; lean_object* x_14; -x_12 = lean_unbox(x_1); -lean_dec(x_1); -x_13 = lean_unbox(x_2); +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_48 = lean_ctor_get(x_18, 1); +lean_inc(x_48); +lean_dec(x_18); +lean_inc(x_15); +x_49 = lean_array_to_list(x_15); +x_50 = lean_box(0); +x_51 = l_List_mapTR_loop___at_Lean_Meta_Match_mkMatcher___spec__6(x_49, x_50); +x_52 = l_Lean_MessageData_ofList(x_51); +x_53 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__2; +x_54 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_54, 0, x_53); +lean_ctor_set(x_54, 1, x_52); +x_55 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__4; +x_56 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_56, 0, x_54); +lean_ctor_set(x_56, 1, x_55); +lean_inc(x_2); +x_57 = l_Lean_MessageData_ofLevel(x_2); +x_58 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_58, 0, x_56); +lean_ctor_set(x_58, 1, x_57); +x_59 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__6; +x_60 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_60, 0, x_58); +lean_ctor_set(x_60, 1, x_59); +lean_inc(x_3); +x_61 = l___private_Init_Data_Repr_0__Nat_reprFast(x_3); +x_62 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_62, 0, x_61); +x_63 = l_Lean_MessageData_ofFormat(x_62); +x_64 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_64, 0, x_60); +lean_ctor_set(x_64, 1, x_63); +x_65 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +x_66 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_66, 0, x_64); +lean_ctor_set(x_66, 1, x_65); +x_67 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_17, x_66, x_7, x_8, x_9, x_10, x_11, x_12, x_48); +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 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__1(x_4, x_5, x_15, x_3, x_2, x_68, x_7, x_8, x_9, x_10, x_11, x_12, x_69); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_68); lean_dec(x_2); -x_14 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1(x_12, x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_6); +lean_dec(x_3); +return x_70; +} +} +} +else +{ +uint8_t x_71; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_5); lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_71 = !lean_is_exclusive(x_14); +if (x_71 == 0) +{ return x_14; } +else +{ +lean_object* x_72; lean_object* x_73; lean_object* x_74; +x_72 = lean_ctor_get(x_14, 0); +x_73 = lean_ctor_get(x_14, 1); +lean_inc(x_73); +lean_inc(x_72); +lean_dec(x_14); +x_74 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_74, 0, x_72); +lean_ctor_set(x_74, 1, x_73); +return x_74; +} } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +} +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___closed__1() { _start: { -uint8_t x_12; uint8_t x_13; lean_object* x_14; -x_12 = lean_unbox(x_1); -lean_dec(x_1); -x_13 = lean_unbox(x_2); +lean_object* x_1; +x_1 = lean_mk_string_unchecked("failed to compute resulting universe level of inductive datatype, provide universe explicitly: ", 95, 95); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_11) == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +x_14 = lean_unsigned_to_nat(0u); +x_15 = l_Lean_Level_getOffsetAux(x_12, x_14); +x_16 = l_Lean_Level_getLevelOffset(x_12); +lean_dec(x_12); +x_17 = l_Lean_Level_isMVar(x_16); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; +lean_dec(x_15); +lean_dec(x_3); lean_dec(x_2); -x_14 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__2(x_12, x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_18 = l_Lean_MessageData_ofLevel(x_16); +x_19 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___closed__2; +x_20 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_20, 0, x_19); +lean_ctor_set(x_20, 1, x_18); +x_21 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +x_22 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_22, 0, x_20); +lean_ctor_set(x_22, 1, x_21); +x_23 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_22, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_24 = !lean_is_exclusive(x_23); +if (x_24 == 0) +{ +return x_23; +} +else +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_23, 0); +x_26 = lean_ctor_get(x_23, 1); +lean_inc(x_26); +lean_inc(x_25); +lean_dec(x_23); +x_27 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +return x_27; +} +} +else +{ +lean_object* x_28; lean_object* x_29; +x_28 = lean_box(0); +x_29 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2(x_1, x_16, x_15, x_2, x_3, x_28, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +return x_29; +} +} +else +{ +uint8_t x_30; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -return x_14; +lean_dec(x_3); +lean_dec(x_2); +x_30 = !lean_is_exclusive(x_11); +if (x_30 == 0) +{ +return x_11; +} +else +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_31 = lean_ctor_get(x_11, 0); +x_32 = lean_ctor_get(x_11, 1); +lean_inc(x_32); +lean_inc(x_31); +lean_dec(x_11); +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_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +} +} +LEAN_EXPORT lean_object* l_Lean_assignLevelMVar___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -uint8_t x_14; uint8_t x_15; uint8_t x_16; uint8_t x_17; lean_object* x_18; -x_14 = lean_unbox(x_1); -lean_dec(x_1); -x_15 = lean_unbox(x_2); -lean_dec(x_2); -x_16 = lean_unbox(x_4); -lean_dec(x_4); -x_17 = lean_unbox(x_5); -lean_dec(x_5); -x_18 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__3(x_14, x_15, x_3, x_16, x_17, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_object* x_10; +x_10 = l_Lean_assignLevelMVar___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -return x_18; +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_10; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -uint8_t x_16; uint8_t x_17; uint8_t x_18; uint8_t x_19; size_t x_20; size_t x_21; lean_object* x_22; -x_16 = lean_unbox(x_1); -lean_dec(x_1); -x_17 = lean_unbox(x_2); -lean_dec(x_2); -x_18 = lean_unbox(x_3); -lean_dec(x_3); -x_19 = lean_unbox(x_4); -lean_dec(x_4); -x_20 = lean_unbox_usize(x_6); -lean_dec(x_6); -x_21 = lean_unbox_usize(x_7); +lean_object* x_10; +x_10 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); lean_dec(x_7); -x_22 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1(x_16, x_17, x_18, x_19, x_5, x_20, x_21, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -lean_dec(x_10); -lean_dec(x_9); +lean_dec(x_6); lean_dec(x_5); -return x_22; +lean_dec(x_4); +lean_dec(x_3); +return x_10; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___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_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -uint8_t x_12; uint8_t x_13; lean_object* x_14; -x_12 = lean_unbox(x_1); -lean_dec(x_1); -x_13 = lean_unbox(x_2); -lean_dec(x_2); -x_14 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__2___lambda__1(x_12, x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_object* x_10; +x_10 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -return x_14; +lean_dec(x_3); +return x_10; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, 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; size_t x_16; size_t x_17; lean_object* x_18; -x_14 = lean_unbox(x_1); -lean_dec(x_1); -x_15 = lean_unbox(x_2); -lean_dec(x_2); -x_16 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_17 = lean_unbox_usize(x_5); -lean_dec(x_5); -x_18 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__2(x_14, x_15, x_3, x_16, x_17, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_object* x_14; +x_14 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_3); -return x_18; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_14; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___boxed(lean_object* x_1, lean_object* x_2, lean_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_Inductive_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -lean_object* x_9; -x_9 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions(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_object* x_14; +x_14 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___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_6); lean_dec(x_1); -return x_9; +return x_14; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getArity___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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_8; lean_object* x_9; -x_8 = lean_array_get_size(x_1); -x_9 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_9, 0, x_8); -lean_ctor_set(x_9, 1, x_7); -return x_9; +lean_object* x_11; +x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_1); +return x_11; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getArity___closed__1() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getArity___lambda__1___boxed), 7, 0); +x_1 = lean_mk_string_unchecked("bootstrap", 9, 9); return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getArity(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__2() { _start: { -lean_object* x_7; lean_object* x_8; uint8_t x_9; lean_object* x_10; -x_7 = lean_ctor_get(x_1, 1); -lean_inc(x_7); -lean_dec(x_1); -x_8 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getArity___closed__1; -x_9 = 0; -x_10 = l_Lean_Meta_forallTelescopeReducing___at_Lean_Meta_getParamNames___spec__2___rarg(x_7, x_8, x_9, x_2, x_3, x_4, x_5, x_6); -return x_10; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("inductiveCheckResultingUniverse", 31, 31); +return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getArity___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__3() { _start: { -lean_object* x_8; -x_8 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getArity___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_8; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__1; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__2; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_resetMaskAt(lean_object* x_1, lean_object* x_2) { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__4() { _start: { -lean_object* x_3; uint8_t x_4; -x_3 = lean_array_get_size(x_1); -x_4 = lean_nat_dec_lt(x_2, x_3); -lean_dec(x_3); -if (x_4 == 0) -{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("by default the `inductive`/`structure` commands report an error if the resulting universe is not zero, but may be zero for some universe parameters. Reason: unless this type is a subsingleton, it is hardly what the user wants since it can only eliminate into `Prop`. In the `Init` package, we define subsingletons, and we use this option to disable the check. This option may be deleted in the future after we improve the validator", 431, 431); return x_1; } -else +} +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__5() { +_start: { -uint8_t x_5; lean_object* x_6; lean_object* x_7; -x_5 = 0; -x_6 = lean_box(x_5); -x_7 = lean_array_fset(x_1, x_2, x_6); -return x_7; +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_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__1; +x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__4; +x_4 = lean_box(x_1); +x_5 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_5, 0, x_4); +lean_ctor_set(x_5, 1, x_2); +lean_ctor_set(x_5, 2, x_3); +return x_5; } } +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__1; +x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__7; +x_4 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__1; +x_5 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__2; +x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); +return x_6; +} } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_resetMaskAt___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753_(lean_object* x_1) { _start: { -lean_object* x_3; -x_3 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_resetMaskAt(x_1, x_2); -lean_dec(x_2); -return x_3; +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__3; +x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__5; +x_4 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__6; +x_5 = l_Lean_Option_register___at_Lean_Elab_initFn____x40_Lean_Elab_AutoBound___hyg_6____spec__1(x_2, x_3, x_4, x_1); +return x_5; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +static lean_object* _init_l_Lean_Elab_Command_checkResultingUniverse___closed__1() { _start: { -uint8_t x_14; -x_14 = lean_nat_dec_le(x_6, x_5); -if (x_14 == 0) +lean_object* x_1; +x_1 = l_Lean_Elab_Command_bootstrap_inductiveCheckResultingUniverse; +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Command_checkResultingUniverse___closed__2() { +_start: { -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_1; +x_1 = lean_mk_string_unchecked("invalid universe polymorphic type, the resultant universe is not Prop (i.e., 0), but it may be Prop for some parameter values (solution: use 'u+1' or 'max 1 u')", 160, 160); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Command_checkResultingUniverse___closed__3() { +_start: { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_25; lean_object* x_36; uint8_t x_37; -lean_dec(x_8); -x_17 = lean_unsigned_to_nat(1u); -x_18 = lean_nat_sub(x_4, x_17); -lean_dec(x_4); -x_36 = lean_array_get_size(x_2); -x_37 = lean_nat_dec_lt(x_5, x_36); -lean_dec(x_36); -if (x_37 == 0) +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_checkResultingUniverse___closed__2; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkResultingUniverse(lean_object* x_1, lean_object* x_2, lean_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_38; -x_38 = lean_box(0); -x_25 = x_38; -goto block_35; +lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_9 = lean_ctor_get(x_6, 2); +x_10 = l_Lean_Elab_Command_checkResultingUniverse___closed__1; +x_11 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_9, x_10); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; +lean_dec(x_2); +lean_dec(x_1); +x_12 = lean_box(0); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_8); +return x_13; } else { -lean_object* x_39; uint8_t x_40; lean_object* x_41; -x_39 = lean_array_get_size(x_3); -x_40 = lean_nat_dec_lt(x_5, x_39); -lean_dec(x_39); -x_41 = lean_array_fget(x_2, x_5); -if (x_40 == 0) +lean_object* x_14; uint8_t x_15; +x_14 = l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_shouldInferResultUniverse___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 0) { -lean_object* x_42; lean_object* x_43; uint8_t x_44; -x_42 = l_Lean_instInhabitedExpr; -x_43 = l_outOfBounds___rarg(x_42); -x_44 = lean_expr_eqv(x_41, x_43); -lean_dec(x_43); -lean_dec(x_41); -if (x_44 == 0) +lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_16 = lean_ctor_get(x_14, 0); +x_17 = lean_ctor_get(x_14, 1); +x_18 = l_Lean_Level_isZero(x_16); +if (x_18 == 0) { -lean_object* x_45; -x_45 = lean_box(0); -x_25 = x_45; -goto block_35; +uint8_t x_19; +x_19 = l_Lean_Level_isNeverZero(x_16); +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_free_object(x_14); +x_20 = l_Lean_MessageData_ofLevel(x_16); +x_21 = l_Lean_indentD(x_20); +x_22 = l_Lean_Elab_Command_checkResultingUniverse___closed__3; +x_23 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_21); +x_24 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +x_25 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +x_26 = l_Lean_throwError___at_Lean_Elab_Term_throwErrorIfErrors___spec__1(x_25, x_2, x_3, x_4, x_5, x_6, x_7, x_17); +return x_26; } else { -lean_object* x_46; -x_46 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; -x_19 = x_46; -x_20 = x_13; -goto block_24; +lean_object* x_27; +lean_dec(x_16); +lean_dec(x_2); +x_27 = lean_box(0); +lean_ctor_set(x_14, 0, x_27); +return x_14; } } else { -lean_object* x_47; uint8_t x_48; -x_47 = lean_array_fget(x_3, x_5); -x_48 = lean_expr_eqv(x_41, x_47); -lean_dec(x_47); -lean_dec(x_41); -if (x_48 == 0) -{ -lean_object* x_49; -x_49 = lean_box(0); -x_25 = x_49; -goto block_35; +lean_object* x_28; +lean_dec(x_16); +lean_dec(x_2); +x_28 = lean_box(0); +lean_ctor_set(x_14, 0, x_28); +return x_14; +} } else { -lean_object* x_50; -x_50 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; -x_19 = x_50; -x_20 = x_13; -goto block_24; -} -} -} -block_24: +lean_object* x_29; lean_object* x_30; uint8_t 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 = l_Lean_Level_isZero(x_29); +if (x_31 == 0) { -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_35: +uint8_t x_32; +x_32 = l_Lean_Level_isNeverZero(x_29); +if (x_32 == 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; lean_object* x_34; -lean_dec(x_25); -x_26 = lean_st_ref_take(x_1, 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 = 0; -x_30 = lean_box(x_29); -x_31 = lean_array_set(x_27, x_5, x_30); -x_32 = lean_st_ref_set(x_1, x_31, x_28); -x_33 = lean_ctor_get(x_32, 1); -lean_inc(x_33); -lean_dec(x_32); -x_34 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; -x_19 = x_34; -x_20 = x_33; -goto block_24; -} +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_MessageData_ofLevel(x_29); +x_34 = l_Lean_indentD(x_33); +x_35 = l_Lean_Elab_Command_checkResultingUniverse___closed__3; +x_36 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_36, 0, x_35); +lean_ctor_set(x_36, 1, x_34); +x_37 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +x_38 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_38, 0, x_36); +lean_ctor_set(x_38, 1, x_37); +x_39 = l_Lean_throwError___at_Lean_Elab_Term_throwErrorIfErrors___spec__1(x_38, x_2, x_3, x_4, x_5, x_6, x_7, x_30); +return x_39; } else { -lean_object* x_51; -lean_dec(x_5); -lean_dec(x_4); -x_51 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_51, 0, x_8); -lean_ctor_set(x_51, 1, x_13); -return x_51; +lean_object* x_40; lean_object* x_41; +lean_dec(x_29); +lean_dec(x_2); +x_40 = lean_box(0); +x_41 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_41, 0, x_40); +lean_ctor_set(x_41, 1, x_30); +return x_41; } } else { -lean_object* x_52; -lean_dec(x_5); -lean_dec(x_4); -x_52 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_52, 0, x_8); -lean_ctor_set(x_52, 1, x_13); -return x_52; -} +lean_object* x_42; lean_object* x_43; +lean_dec(x_29); +lean_dec(x_2); +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_30); +return x_43; } } -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___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; lean_object* x_7; uint8_t x_8; -x_6 = lean_array_uget(x_2, x_3); -x_7 = l_Lean_Expr_getAppFn(x_1); -x_8 = lean_expr_eqv(x_7, x_6); -lean_dec(x_6); -lean_dec(x_7); -if (x_8 == 0) -{ -size_t x_9; size_t x_10; -x_9 = 1; -x_10 = lean_usize_add(x_3, x_9); -x_3 = x_10; -goto _start; } -else -{ -uint8_t x_12; -x_12 = 1; -return x_12; } } -else +LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkResultingUniverse___boxed(lean_object* x_1, lean_object* x_2, lean_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 = 0; -return x_13; -} +lean_object* x_9; +x_9 = l_Lean_Elab_Command_checkResultingUniverse(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_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { uint8_t x_15; -x_15 = lean_nat_dec_le(x_7, x_6); +x_15 = lean_usize_dec_lt(x_6, x_5); 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_27; uint8_t x_28; +lean_object* x_16; +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); 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_27 = lean_array_get_size(x_2); -x_28 = lean_nat_dec_le(x_27, x_6); -if (x_28 == 0) -{ -uint8_t x_29; uint8_t x_30; -x_29 = lean_nat_dec_lt(x_6, x_4); -x_30 = lean_nat_dec_lt(x_6, x_27); -lean_dec(x_27); -if (x_29 == 0) -{ -lean_object* x_31; lean_object* x_32; -x_31 = l_Lean_instInhabitedExpr; -x_32 = l_outOfBounds___rarg(x_31); -if (x_30 == 0) +lean_dec(x_8); +lean_dec(x_3); +lean_dec(x_2); +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_7); +lean_ctor_set(x_16, 1, x_14); +return x_16; +} +else { -lean_object* x_33; uint8_t x_34; -x_33 = l_outOfBounds___rarg(x_31); -x_34 = lean_expr_eqv(x_32, x_33); -lean_dec(x_33); -lean_dec(x_32); -if (x_34 == 0) +lean_object* x_17; lean_object* x_18; uint8_t x_19; +lean_dec(x_7); +x_17 = lean_array_uget(x_4, x_6); +x_18 = lean_ctor_get(x_17, 2); +lean_inc(x_18); +x_19 = lean_name_eq(x_18, x_1); +lean_dec(x_18); +if (x_19 == 0) { -lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; -x_35 = lean_st_ref_take(x_1, x_14); -x_36 = lean_ctor_get(x_35, 0); -lean_inc(x_36); -x_37 = lean_ctor_get(x_35, 1); -lean_inc(x_37); -lean_dec(x_35); -x_38 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_resetMaskAt(x_36, x_6); -x_39 = lean_st_ref_set(x_1, x_38, x_37); -x_40 = !lean_is_exclusive(x_39); -if (x_40 == 0) +size_t x_20; size_t x_21; +lean_dec(x_17); +x_20 = 1; +x_21 = lean_usize_add(x_6, x_20); +lean_inc(x_3); { -lean_object* x_41; lean_object* x_42; -x_41 = lean_ctor_get(x_39, 0); -lean_dec(x_41); -x_42 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; -lean_ctor_set(x_39, 0, x_42); -x_20 = x_39; -goto block_26; +size_t _tmp_5 = x_21; +lean_object* _tmp_6 = x_3; +x_6 = _tmp_5; +x_7 = _tmp_6; +} +goto _start; } else { -lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_43 = lean_ctor_get(x_39, 1); -lean_inc(x_43); -lean_dec(x_39); -x_44 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; -x_45 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_45, 0, x_44); -lean_ctor_set(x_45, 1, x_43); -x_20 = x_45; -goto block_26; -} +lean_object* x_23; uint8_t x_24; +lean_dec(x_3); +x_23 = lean_ctor_get(x_17, 0); +lean_inc(x_23); +lean_dec(x_17); +x_24 = !lean_is_exclusive(x_12); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_12, 5); +x_26 = l_Lean_replaceRef(x_23, x_25); +lean_dec(x_25); +lean_dec(x_23); +lean_ctor_set(x_12, 5, x_26); +x_27 = lean_apply_7(x_2, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +if (lean_obj_tag(x_27) == 0) +{ +uint8_t x_28; +x_28 = !lean_is_exclusive(x_27); +if (x_28 == 0) +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_29 = lean_ctor_get(x_27, 0); +x_30 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_30, 0, x_29); +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_27, 0, x_32); +return x_27; } else { -lean_object* x_46; lean_object* x_47; -x_46 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; -x_47 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_47, 0, x_46); -lean_ctor_set(x_47, 1, x_14); -x_20 = x_47; -goto block_26; +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_33 = lean_ctor_get(x_27, 0); +x_34 = lean_ctor_get(x_27, 1); +lean_inc(x_34); +lean_inc(x_33); +lean_dec(x_27); +x_35 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_35, 0, x_33); +x_36 = lean_box(0); +x_37 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +x_38 = lean_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_48; uint8_t x_49; -x_48 = lean_array_fget(x_2, x_6); -x_49 = lean_expr_eqv(x_32, x_48); -lean_dec(x_48); -lean_dec(x_32); -if (x_49 == 0) -{ -lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; uint8_t x_55; -x_50 = lean_st_ref_take(x_1, x_14); -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_Inductive_0__Lean_Elab_Command_resetMaskAt(x_51, x_6); -x_54 = lean_st_ref_set(x_1, x_53, x_52); -x_55 = !lean_is_exclusive(x_54); -if (x_55 == 0) +uint8_t x_39; +x_39 = !lean_is_exclusive(x_27); +if (x_39 == 0) { -lean_object* x_56; lean_object* x_57; -x_56 = lean_ctor_get(x_54, 0); -lean_dec(x_56); -x_57 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; -lean_ctor_set(x_54, 0, x_57); -x_20 = x_54; -goto block_26; +return x_27; } else { -lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_58 = lean_ctor_get(x_54, 1); -lean_inc(x_58); -lean_dec(x_54); -x_59 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; -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_20 = x_60; -goto block_26; +lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_40 = lean_ctor_get(x_27, 0); +x_41 = lean_ctor_get(x_27, 1); +lean_inc(x_41); +lean_inc(x_40); +lean_dec(x_27); +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_61; lean_object* x_62; -x_61 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; -x_62 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_62, 0, x_61); -lean_ctor_set(x_62, 1, x_14); -x_20 = x_62; -goto block_26; +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; uint8_t x_54; lean_object* x_55; uint8_t x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_43 = lean_ctor_get(x_12, 0); +x_44 = lean_ctor_get(x_12, 1); +x_45 = lean_ctor_get(x_12, 2); +x_46 = lean_ctor_get(x_12, 3); +x_47 = lean_ctor_get(x_12, 4); +x_48 = lean_ctor_get(x_12, 5); +x_49 = lean_ctor_get(x_12, 6); +x_50 = lean_ctor_get(x_12, 7); +x_51 = lean_ctor_get(x_12, 8); +x_52 = lean_ctor_get(x_12, 9); +x_53 = lean_ctor_get(x_12, 10); +x_54 = lean_ctor_get_uint8(x_12, sizeof(void*)*12); +x_55 = lean_ctor_get(x_12, 11); +x_56 = lean_ctor_get_uint8(x_12, sizeof(void*)*12 + 1); +lean_inc(x_55); +lean_inc(x_53); +lean_inc(x_52); +lean_inc(x_51); +lean_inc(x_50); +lean_inc(x_49); +lean_inc(x_48); +lean_inc(x_47); +lean_inc(x_46); +lean_inc(x_45); +lean_inc(x_44); +lean_inc(x_43); +lean_dec(x_12); +x_57 = l_Lean_replaceRef(x_23, x_48); +lean_dec(x_48); +lean_dec(x_23); +x_58 = lean_alloc_ctor(0, 12, 2); +lean_ctor_set(x_58, 0, x_43); +lean_ctor_set(x_58, 1, x_44); +lean_ctor_set(x_58, 2, x_45); +lean_ctor_set(x_58, 3, x_46); +lean_ctor_set(x_58, 4, x_47); +lean_ctor_set(x_58, 5, x_57); +lean_ctor_set(x_58, 6, x_49); +lean_ctor_set(x_58, 7, x_50); +lean_ctor_set(x_58, 8, x_51); +lean_ctor_set(x_58, 9, x_52); +lean_ctor_set(x_58, 10, x_53); +lean_ctor_set(x_58, 11, x_55); +lean_ctor_set_uint8(x_58, sizeof(void*)*12, x_54); +lean_ctor_set_uint8(x_58, sizeof(void*)*12 + 1, x_56); +x_59 = lean_apply_7(x_2, x_8, x_9, x_10, x_11, x_58, x_13, x_14); +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; lean_object* x_65; lean_object* x_66; +x_60 = lean_ctor_get(x_59, 0); +lean_inc(x_60); +x_61 = lean_ctor_get(x_59, 1); +lean_inc(x_61); +if (lean_is_exclusive(x_59)) { + lean_ctor_release(x_59, 0); + lean_ctor_release(x_59, 1); + x_62 = x_59; +} else { + lean_dec_ref(x_59); + x_62 = lean_box(0); } +x_63 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_63, 0, x_60); +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); +if (lean_is_scalar(x_62)) { + x_66 = lean_alloc_ctor(0, 2, 0); +} else { + x_66 = x_62; } +lean_ctor_set(x_66, 0, x_65); +lean_ctor_set(x_66, 1, x_61); +return x_66; } else { -lean_object* x_63; -x_63 = lean_array_fget(x_3, x_6); -if (x_30 == 0) -{ -lean_object* x_64; lean_object* x_65; uint8_t x_66; -x_64 = l_Lean_instInhabitedExpr; -x_65 = l_outOfBounds___rarg(x_64); -x_66 = lean_expr_eqv(x_63, x_65); -lean_dec(x_65); -lean_dec(x_63); -if (x_66 == 0) -{ -lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; uint8_t x_72; -x_67 = lean_st_ref_take(x_1, x_14); -x_68 = lean_ctor_get(x_67, 0); +lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; +x_67 = lean_ctor_get(x_59, 0); +lean_inc(x_67); +x_68 = lean_ctor_get(x_59, 1); lean_inc(x_68); -x_69 = lean_ctor_get(x_67, 1); -lean_inc(x_69); -lean_dec(x_67); -x_70 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_resetMaskAt(x_68, x_6); -x_71 = lean_st_ref_set(x_1, x_70, x_69); -x_72 = !lean_is_exclusive(x_71); -if (x_72 == 0) -{ -lean_object* x_73; lean_object* x_74; -x_73 = lean_ctor_get(x_71, 0); -lean_dec(x_73); -x_74 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; -lean_ctor_set(x_71, 0, x_74); -x_20 = x_71; -goto block_26; +if (lean_is_exclusive(x_59)) { + lean_ctor_release(x_59, 0); + lean_ctor_release(x_59, 1); + x_69 = x_59; +} else { + lean_dec_ref(x_59); + x_69 = lean_box(0); } -else -{ -lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_75 = lean_ctor_get(x_71, 1); -lean_inc(x_75); -lean_dec(x_71); -x_76 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; -x_77 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_77, 0, x_76); -lean_ctor_set(x_77, 1, x_75); -x_20 = x_77; -goto block_26; +if (lean_is_scalar(x_69)) { + x_70 = lean_alloc_ctor(1, 2, 0); +} else { + x_70 = x_69; } +lean_ctor_set(x_70, 0, x_67); +lean_ctor_set(x_70, 1, x_68); +return x_70; } -else -{ -lean_object* x_78; lean_object* x_79; -x_78 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; -x_79 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_79, 0, x_78); -lean_ctor_set(x_79, 1, x_14); -x_20 = x_79; -goto block_26; } } -else -{ -lean_object* x_80; uint8_t x_81; -x_80 = lean_array_fget(x_2, x_6); -x_81 = lean_expr_eqv(x_63, x_80); -lean_dec(x_80); -lean_dec(x_63); -if (x_81 == 0) -{ -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_82 = lean_st_ref_take(x_1, x_14); -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 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_resetMaskAt(x_83, x_6); -x_86 = lean_st_ref_set(x_1, x_85, x_84); -x_87 = !lean_is_exclusive(x_86); -if (x_87 == 0) -{ -lean_object* x_88; lean_object* x_89; -x_88 = lean_ctor_get(x_86, 0); -lean_dec(x_88); -x_89 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; -lean_ctor_set(x_86, 0, x_89); -x_20 = x_86; -goto block_26; } -else +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: { -lean_object* x_90; lean_object* x_91; lean_object* x_92; -x_90 = lean_ctor_get(x_86, 1); -lean_inc(x_90); -lean_dec(x_86); -x_91 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; -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_20 = x_92; -goto block_26; -} -} -else -{ -lean_object* x_93; lean_object* x_94; -x_93 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; -x_94 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_94, 0, x_93); -lean_ctor_set(x_94, 1, x_14); -x_20 = x_94; -goto block_26; -} -} -} -} -else -{ -lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; uint8_t x_100; -lean_dec(x_27); -x_95 = lean_st_ref_take(x_1, x_14); -x_96 = lean_ctor_get(x_95, 0); -lean_inc(x_96); -x_97 = lean_ctor_get(x_95, 1); -lean_inc(x_97); -lean_dec(x_95); -x_98 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_resetMaskAt(x_96, x_6); -x_99 = lean_st_ref_set(x_1, x_98, x_97); -x_100 = !lean_is_exclusive(x_99); -if (x_100 == 0) +uint8_t x_15; +x_15 = lean_usize_dec_lt(x_6, x_5); +if (x_15 == 0) { -lean_object* x_101; lean_object* x_102; -x_101 = lean_ctor_get(x_99, 0); -lean_dec(x_101); -x_102 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; -lean_ctor_set(x_99, 0, x_102); -x_20 = x_99; -goto block_26; +lean_object* 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_3); +lean_dec(x_2); +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_7); +lean_ctor_set(x_16, 1, x_14); +return x_16; } else { -lean_object* x_103; lean_object* x_104; lean_object* x_105; -x_103 = lean_ctor_get(x_99, 1); -lean_inc(x_103); -lean_dec(x_99); -x_104 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; -x_105 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_105, 0, x_104); -lean_ctor_set(x_105, 1, x_103); -x_20 = x_105; -goto block_26; -} -} -block_26: +lean_object* x_17; lean_object* x_18; size_t x_19; size_t x_20; lean_object* x_21; +lean_dec(x_7); +x_17 = lean_array_uget(x_4, x_6); +x_18 = lean_ctor_get(x_17, 8); +lean_inc(x_18); +lean_dec(x_17); +x_19 = lean_array_size(x_18); +x_20 = 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); +lean_inc_n(x_3, 2); +lean_inc(x_2); +x_21 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___spec__2(x_1, x_2, x_3, x_18, x_19, x_20, x_3, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_18); +if (lean_obj_tag(x_21) == 0) { -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_20, 1); +lean_object* x_22; lean_object* x_23; +x_22 = lean_ctor_get(x_21, 0); lean_inc(x_22); -lean_dec(x_20); -x_23 = lean_ctor_get(x_21, 0); +x_23 = lean_ctor_get(x_22, 0); lean_inc(x_23); +lean_dec(x_22); +if (lean_obj_tag(x_23) == 0) +{ +lean_object* x_24; size_t x_25; size_t x_26; +x_24 = lean_ctor_get(x_21, 1); +lean_inc(x_24); lean_dec(x_21); -x_24 = lean_nat_add(x_6, x_8); -lean_dec(x_6); -x_5 = x_19; -x_6 = x_24; -x_9 = x_23; -x_14 = x_22; +x_25 = 1; +x_26 = lean_usize_add(x_6, x_25); +lean_inc(x_3); +{ +size_t _tmp_5 = x_26; +lean_object* _tmp_6 = x_3; +lean_object* _tmp_13 = x_24; +x_6 = _tmp_5; +x_7 = _tmp_6; +x_14 = _tmp_13; +} goto _start; } +else +{ +uint8_t x_28; +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_3); +lean_dec(x_2); +x_28 = !lean_is_exclusive(x_21); +if (x_28 == 0) +{ +lean_object* x_29; uint8_t x_30; +x_29 = lean_ctor_get(x_21, 0); +lean_dec(x_29); +x_30 = !lean_is_exclusive(x_23); +if (x_30 == 0) +{ +lean_object* x_31; lean_object* x_32; +x_31 = lean_box(0); +x_32 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_32, 0, x_23); +lean_ctor_set(x_32, 1, x_31); +lean_ctor_set(x_21, 0, x_32); +return x_21; } else { -lean_object* x_106; -lean_dec(x_6); -lean_dec(x_5); -x_106 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_106, 0, x_9); -lean_ctor_set(x_106, 1, x_14); -return x_106; +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_box(0); +x_36 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_36, 0, x_34); +lean_ctor_set(x_36, 1, x_35); +lean_ctor_set(x_21, 0, x_36); +return x_21; } } else { -lean_object* x_107; -lean_dec(x_6); -lean_dec(x_5); -x_107 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_107, 0, x_9); -lean_ctor_set(x_107, 1, x_14); -return x_107; +lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_37 = lean_ctor_get(x_21, 1); +lean_inc(x_37); +lean_dec(x_21); +x_38 = lean_ctor_get(x_23, 0); +lean_inc(x_38); +if (lean_is_exclusive(x_23)) { + lean_ctor_release(x_23, 0); + x_39 = x_23; +} else { + lean_dec_ref(x_23); + x_39 = lean_box(0); +} +if (lean_is_scalar(x_39)) { + x_40 = lean_alloc_ctor(1, 1, 0); +} else { + x_40 = x_39; } +lean_ctor_set(x_40, 0, x_38); +x_41 = lean_box(0); +x_42 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_42, 0, x_40); +lean_ctor_set(x_42, 1, x_41); +x_43 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_43, 0, x_42); +lean_ctor_set(x_43, 1, x_37); +return x_43; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___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) { -_start: -{ -uint8_t x_12; -x_12 = lean_nat_dec_le(x_4, x_3); -if (x_12 == 0) -{ -lean_object* x_13; uint8_t x_14; -x_13 = lean_unsigned_to_nat(0u); -x_14 = lean_nat_dec_eq(x_2, x_13); -if (x_14 == 0) -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; -lean_dec(x_6); -x_15 = lean_unsigned_to_nat(1u); -x_16 = lean_nat_sub(x_2, x_15); -lean_dec(x_2); -x_17 = lean_st_ref_take(x_1, 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_20 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_resetMaskAt(x_18, x_3); -x_21 = lean_st_ref_set(x_1, x_20, x_19); -x_22 = lean_ctor_get(x_21, 1); -lean_inc(x_22); -lean_dec(x_21); -x_23 = lean_nat_add(x_3, x_5); -lean_dec(x_3); -x_24 = lean_box(0); -x_2 = x_16; -x_3 = x_23; -x_6 = x_24; -x_11 = x_22; -goto _start; } else { -lean_object* x_26; +uint8_t x_44; +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); lean_dec(x_3); lean_dec(x_2); -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_6); -lean_ctor_set(x_26, 1, x_11); -return x_26; -} +x_44 = !lean_is_exclusive(x_21); +if (x_44 == 0) +{ +return x_21; } else { -lean_object* x_27; -lean_dec(x_3); -lean_dec(x_2); -x_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_6); -lean_ctor_set(x_27, 1, x_11); -return x_27; +lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_45 = lean_ctor_get(x_21, 0); +x_46 = lean_ctor_get(x_21, 1); +lean_inc(x_46); +lean_inc(x_45); +lean_dec(x_21); +x_47 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_47, 0, x_45); +lean_ctor_set(x_47, 1, x_46); +return x_47; } } } -LEAN_EXPORT lean_object* l_Lean_ForEachExprWhere_visited___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_withCtorRef___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___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_8; uint8_t x_9; -x_8 = lean_st_ref_get(x_2, x_7); -x_9 = !lean_is_exclusive(x_8); -if (x_9 == 0) +lean_object* x_10; +x_10 = lean_apply_7(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_withCtorRef___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___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_10; lean_object* x_11; size_t x_12; size_t x_13; size_t x_14; lean_object* x_15; lean_object* x_16; size_t x_17; uint8_t x_18; -x_10 = lean_ctor_get(x_8, 0); -x_11 = lean_ctor_get(x_8, 1); -x_12 = lean_ptr_addr(x_1); -x_13 = 8191; -x_14 = lean_usize_mod(x_12, x_13); -x_15 = lean_ctor_get(x_10, 0); +size_t x_11; size_t x_12; lean_object* x_13; lean_object* x_14; +x_11 = lean_array_size(x_1); +x_12 = 0; +x_13 = l_Lean_Elab_Command_withCtorRef___rarg___closed__1; +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_14 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___spec__3(x_2, x_3, x_13, x_1, x_11, x_12, x_13, 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; +x_15 = lean_ctor_get(x_14, 0); lean_inc(x_15); -lean_dec(x_10); -x_16 = lean_array_uget(x_15, x_14); +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); lean_dec(x_15); -x_17 = lean_ptr_addr(x_16); -lean_dec(x_16); -x_18 = lean_usize_dec_eq(x_17, x_12); -if (x_18 == 0) +if (lean_obj_tag(x_16) == 0) { -lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; -lean_free_object(x_8); -x_19 = lean_st_ref_take(x_2, x_11); -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_19, 1); -lean_inc(x_21); -lean_dec(x_19); -x_22 = !lean_is_exclusive(x_20); -if (x_22 == 0) +lean_object* x_17; lean_object* x_18; +x_17 = lean_ctor_get(x_14, 1); +lean_inc(x_17); +lean_dec(x_14); +x_18 = lean_apply_7(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_17); +return x_18; +} +else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; -x_23 = lean_ctor_get(x_20, 0); -x_24 = lean_array_uset(x_23, x_14, x_1); -lean_ctor_set(x_20, 0, x_24); -x_25 = lean_st_ref_set(x_2, x_20, x_21); -x_26 = !lean_is_exclusive(x_25); -if (x_26 == 0) +uint8_t x_19; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_19 = !lean_is_exclusive(x_14); +if (x_19 == 0) { -lean_object* x_27; uint8_t x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_25, 0); -lean_dec(x_27); -x_28 = 0; -x_29 = lean_box(x_28); -lean_ctor_set(x_25, 0, x_29); -return x_25; +lean_object* x_20; lean_object* x_21; +x_20 = lean_ctor_get(x_14, 0); +lean_dec(x_20); +x_21 = lean_ctor_get(x_16, 0); +lean_inc(x_21); +lean_dec(x_16); +lean_ctor_set(x_14, 0, x_21); +return x_14; } else { -lean_object* x_30; uint8_t x_31; lean_object* x_32; lean_object* x_33; -x_30 = lean_ctor_get(x_25, 1); -lean_inc(x_30); -lean_dec(x_25); -x_31 = 0; -x_32 = lean_box(x_31); -x_33 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_33, 0, x_32); -lean_ctor_set(x_33, 1, x_30); -return x_33; +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_14, 1); +lean_inc(x_22); +lean_dec(x_14); +x_23 = lean_ctor_get(x_16, 0); +lean_inc(x_23); +lean_dec(x_16); +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_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; lean_object* x_42; lean_object* x_43; -x_34 = lean_ctor_get(x_20, 0); -x_35 = lean_ctor_get(x_20, 1); -lean_inc(x_35); -lean_inc(x_34); -lean_dec(x_20); -x_36 = lean_array_uset(x_34, x_14, x_1); -x_37 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_37, 0, x_36); -lean_ctor_set(x_37, 1, x_35); -x_38 = lean_st_ref_set(x_2, x_37, x_21); -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); +uint8_t x_25; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_25 = !lean_is_exclusive(x_14); +if (x_25 == 0) +{ +return x_14; } -x_41 = 0; -x_42 = lean_box(x_41); -if (lean_is_scalar(x_40)) { - x_43 = lean_alloc_ctor(0, 2, 0); -} else { - x_43 = x_40; +else +{ +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_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; } -lean_ctor_set(x_43, 0, x_42); -lean_ctor_set(x_43, 1, x_39); -return x_43; } } -else +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1___closed__1() { +_start: { -uint8_t x_44; lean_object* x_45; -lean_dec(x_1); -x_44 = 1; -x_45 = lean_box(x_44); -lean_ctor_set(x_8, 0, x_45); -return x_8; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("\nat universe level", 18, 18); +return x_1; } } -else -{ -lean_object* x_46; lean_object* x_47; size_t x_48; size_t x_49; size_t x_50; lean_object* x_51; lean_object* x_52; size_t x_53; uint8_t x_54; -x_46 = lean_ctor_get(x_8, 0); -x_47 = lean_ctor_get(x_8, 1); -lean_inc(x_47); -lean_inc(x_46); -lean_dec(x_8); -x_48 = lean_ptr_addr(x_1); -x_49 = 8191; -x_50 = lean_usize_mod(x_48, x_49); -x_51 = lean_ctor_get(x_46, 0); -lean_inc(x_51); -lean_dec(x_46); -x_52 = lean_array_uget(x_51, x_50); -lean_dec(x_51); -x_53 = lean_ptr_addr(x_52); -lean_dec(x_52); -x_54 = lean_usize_dec_eq(x_53, x_48); -if (x_54 == 0) +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1___closed__2() { +_start: { -lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; uint8_t x_66; lean_object* x_67; lean_object* x_68; -x_55 = lean_st_ref_take(x_2, x_47); -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); -x_59 = lean_ctor_get(x_56, 1); -lean_inc(x_59); -if (lean_is_exclusive(x_56)) { - lean_ctor_release(x_56, 0); - lean_ctor_release(x_56, 1); - x_60 = x_56; -} else { - lean_dec_ref(x_56); - x_60 = lean_box(0); +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } -x_61 = lean_array_uset(x_58, x_50, x_1); -if (lean_is_scalar(x_60)) { - x_62 = lean_alloc_ctor(0, 2, 0); -} else { - x_62 = x_60; } -lean_ctor_set(x_62, 0, x_61); -lean_ctor_set(x_62, 1, x_59); -x_63 = lean_st_ref_set(x_2, x_62, x_57); -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 = 0; -x_67 = lean_box(x_66); -if (lean_is_scalar(x_65)) { - x_68 = lean_alloc_ctor(0, 2, 0); -} else { - x_68 = x_65; +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("\nit must be smaller than or equal to the inductive datatype universe level", 74, 74); +return x_1; } -lean_ctor_set(x_68, 0, x_67); -lean_ctor_set(x_68, 1, x_64); -return x_68; } -else +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1___closed__4() { +_start: { -uint8_t x_69; lean_object* x_70; lean_object* x_71; -lean_dec(x_1); -x_69 = 1; -x_70 = lean_box(x_69); -x_71 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_71, 0, x_70); -lean_ctor_set(x_71, 1, x_47); -return x_71; +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; 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_15 = l_Lean_indentExpr(x_1); +x_16 = l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__2; +x_17 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_17, 0, x_16); +lean_ctor_set(x_17, 1, x_15); +x_18 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +x_19 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set(x_19, 1, x_18); +x_20 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_20, 0, x_6); +lean_ctor_set(x_20, 1, x_19); +x_21 = l_Lean_MessageData_ofLevel(x_2); +x_22 = l_Lean_indentD(x_21); +x_23 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1___closed__2; +x_24 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_24, 0, x_23); +lean_ctor_set(x_24, 1, x_22); +x_25 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_25, 0, x_24); +lean_ctor_set(x_25, 1, x_18); +x_26 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_26, 0, x_20); +lean_ctor_set(x_26, 1, x_25); +x_27 = l_Lean_MessageData_ofLevel(x_3); +x_28 = l_Lean_indentD(x_27); +x_29 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1___closed__4; +x_30 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_30, 0, x_29); +lean_ctor_set(x_30, 1, x_28); +x_31 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_31, 0, x_30); +lean_ctor_set(x_31, 1, x_18); +x_32 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_32, 0, x_26); +lean_ctor_set(x_32, 1, x_31); +x_33 = lean_alloc_closure((void*)(l_Lean_throwError___at_Lean_Elab_Term_throwErrorIfErrors___spec__1___boxed), 8, 1); +lean_closure_set(x_33, 0, x_32); +x_34 = l_Lean_Elab_Command_withCtorRef___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___spec__1(x_4, x_5, x_33, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +return x_34; } } -LEAN_EXPORT lean_object* l_Lean_ForEachExprWhere_checked___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___closed__1() { _start: { -lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; -x_8 = lean_st_ref_get(x_2, x_7); -x_9 = lean_ctor_get(x_8, 0); -lean_inc(x_9); -x_10 = lean_ctor_get(x_9, 1); -lean_inc(x_10); -lean_dec(x_9); -x_11 = !lean_is_exclusive(x_8); -if (x_11 == 0) -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint64_t x_16; uint64_t x_17; uint64_t x_18; uint64_t x_19; uint64_t x_20; uint64_t x_21; uint64_t x_22; size_t x_23; size_t x_24; size_t x_25; size_t x_26; size_t x_27; lean_object* x_28; uint8_t x_29; -x_12 = lean_ctor_get(x_8, 1); -x_13 = lean_ctor_get(x_8, 0); -lean_dec(x_13); -x_14 = lean_ctor_get(x_10, 1); -lean_inc(x_14); -lean_dec(x_10); -x_15 = lean_array_get_size(x_14); -x_16 = l_Lean_Expr_hash(x_1); -x_17 = 32; -x_18 = lean_uint64_shift_right(x_16, x_17); -x_19 = lean_uint64_xor(x_16, x_18); -x_20 = 16; -x_21 = lean_uint64_shift_right(x_19, x_20); -x_22 = lean_uint64_xor(x_19, x_21); -x_23 = lean_uint64_to_usize(x_22); -x_24 = lean_usize_of_nat(x_15); -lean_dec(x_15); -x_25 = 1; -x_26 = lean_usize_sub(x_24, x_25); -x_27 = lean_usize_land(x_23, x_26); -x_28 = lean_array_uget(x_14, x_27); -lean_dec(x_14); -x_29 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_CollectLevelMVars_visitExpr___spec__1(x_1, x_28); -lean_dec(x_28); -if (x_29 == 0) -{ -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; -lean_free_object(x_8); -x_30 = lean_st_ref_take(x_2, x_12); -x_31 = lean_ctor_get(x_30, 0); -lean_inc(x_31); -x_32 = lean_ctor_get(x_31, 1); -lean_inc(x_32); -x_33 = lean_ctor_get(x_30, 1); -lean_inc(x_33); -lean_dec(x_30); -x_34 = !lean_is_exclusive(x_31); -if (x_34 == 0) -{ -lean_object* x_35; uint8_t x_36; -x_35 = lean_ctor_get(x_31, 1); -lean_dec(x_35); -x_36 = !lean_is_exclusive(x_32); -if (x_36 == 0) -{ -lean_object* x_37; lean_object* x_38; lean_object* x_39; size_t x_40; size_t x_41; size_t x_42; lean_object* x_43; uint8_t x_44; -x_37 = lean_ctor_get(x_32, 0); -x_38 = lean_ctor_get(x_32, 1); -x_39 = lean_array_get_size(x_38); -x_40 = lean_usize_of_nat(x_39); -lean_dec(x_39); -x_41 = lean_usize_sub(x_40, x_25); -x_42 = lean_usize_land(x_23, x_41); -x_43 = lean_array_uget(x_38, x_42); -x_44 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_CollectLevelMVars_visitExpr___spec__1(x_1, x_43); -if (x_44 == 0) -{ -lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; uint8_t x_55; -x_45 = lean_unsigned_to_nat(1u); -x_46 = lean_nat_add(x_37, x_45); -lean_dec(x_37); -x_47 = lean_box(0); -x_48 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_48, 0, x_1); -lean_ctor_set(x_48, 1, x_47); -lean_ctor_set(x_48, 2, x_43); -x_49 = lean_array_uset(x_38, x_42, x_48); -x_50 = lean_unsigned_to_nat(4u); -x_51 = lean_nat_mul(x_46, x_50); -x_52 = lean_unsigned_to_nat(3u); -x_53 = lean_nat_div(x_51, x_52); -lean_dec(x_51); -x_54 = lean_array_get_size(x_49); -x_55 = lean_nat_dec_le(x_53, x_54); -lean_dec(x_54); -lean_dec(x_53); -if (x_55 == 0) -{ -lean_object* x_56; lean_object* x_57; uint8_t x_58; -x_56 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_CollectLevelMVars_visitExpr___spec__2(x_49); -lean_ctor_set(x_32, 1, x_56); -lean_ctor_set(x_32, 0, x_46); -x_57 = lean_st_ref_set(x_2, x_31, x_33); -x_58 = !lean_is_exclusive(x_57); -if (x_58 == 0) -{ -lean_object* x_59; uint8_t x_60; lean_object* x_61; -x_59 = lean_ctor_get(x_57, 0); -lean_dec(x_59); -x_60 = 0; -x_61 = lean_box(x_60); -lean_ctor_set(x_57, 0, x_61); -return x_57; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("invalid universe level in constructor '", 39, 39); +return x_1; } -else +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___closed__2() { +_start: { -lean_object* x_62; uint8_t x_63; lean_object* x_64; lean_object* x_65; -x_62 = lean_ctor_get(x_57, 1); -lean_inc(x_62); -lean_dec(x_57); -x_63 = 0; -x_64 = lean_box(x_63); -x_65 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_65, 0, x_64); -lean_ctor_set(x_65, 1, x_62); -return x_65; +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -else -{ -lean_object* x_66; uint8_t x_67; -lean_ctor_set(x_32, 1, x_49); -lean_ctor_set(x_32, 0, x_46); -x_66 = lean_st_ref_set(x_2, x_31, x_33); -x_67 = !lean_is_exclusive(x_66); -if (x_67 == 0) +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___closed__3() { +_start: { -lean_object* x_68; uint8_t x_69; lean_object* x_70; -x_68 = lean_ctor_get(x_66, 0); -lean_dec(x_68); -x_69 = 0; -x_70 = lean_box(x_69); -lean_ctor_set(x_66, 0, x_70); -return x_66; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("', parameter", 12, 12); +return x_1; } -else +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___closed__4() { +_start: { -lean_object* x_71; uint8_t x_72; lean_object* x_73; lean_object* x_74; -x_71 = lean_ctor_get(x_66, 1); -lean_inc(x_71); -lean_dec(x_66); -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_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_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, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +_start: +{ +switch (lean_obj_tag(x_7)) { +case 1: +{ +if (lean_obj_tag(x_8) == 1) +{ +lean_object* x_16; lean_object* x_17; +x_16 = lean_ctor_get(x_7, 0); +lean_inc(x_16); +lean_dec(x_7); +x_17 = lean_ctor_get(x_8, 0); +lean_inc(x_17); +lean_dec(x_8); +x_7 = x_16; +x_8 = x_17; +goto _start; } else { -lean_object* x_75; uint8_t x_76; -lean_dec(x_43); -lean_dec(x_1); -x_75 = lean_st_ref_set(x_2, x_31, x_33); -x_76 = !lean_is_exclusive(x_75); -if (x_76 == 0) +uint8_t x_19; +lean_dec(x_8); +lean_dec(x_7); +x_19 = l_Lean_Level_geq(x_2, x_6); +if (x_19 == 0) { -lean_object* x_77; uint8_t x_78; lean_object* x_79; -x_77 = lean_ctor_get(x_75, 0); -lean_dec(x_77); -x_78 = 0; -x_79 = lean_box(x_78); -lean_ctor_set(x_75, 0, x_79); -return x_75; +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_3, 0); +lean_inc(x_20); +lean_dec(x_3); +lean_inc(x_20); +x_21 = l_Lean_MessageData_ofName(x_20); +x_22 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___closed__2; +x_23 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_21); +x_24 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___closed__4; +x_25 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +lean_inc(x_11); +x_26 = l_Lean_Meta_getFVarLocalDecl(x_4, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_26) == 0) +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; +x_27 = lean_ctor_get(x_26, 0); +lean_inc(x_27); +x_28 = lean_ctor_get(x_26, 1); +lean_inc(x_28); +lean_dec(x_26); +x_29 = l_Lean_LocalDecl_userName(x_27); +lean_dec(x_27); +x_30 = l_Lean_Name_hasMacroScopes(x_29); +lean_dec(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; +x_31 = l_Lean_MessageData_ofExpr(x_4); +x_32 = l_Lean_Elab_Command_accLevelAtCtor___closed__8; +x_33 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_31); +x_34 = l_Lean_Elab_Command_accLevelAtCtor___closed__10; +x_35 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +x_36 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_36, 0, x_25); +lean_ctor_set(x_36, 1, x_35); +x_37 = lean_box(0); +x_38 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1(x_5, x_6, x_2, x_1, x_20, x_36, x_37, x_9, x_10, x_11, x_12, x_13, x_14, x_28); +lean_dec(x_20); +return x_38; } else { -lean_object* x_80; uint8_t x_81; lean_object* x_82; lean_object* x_83; -x_80 = lean_ctor_get(x_75, 1); -lean_inc(x_80); -lean_dec(x_75); -x_81 = 0; -x_82 = lean_box(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_80); -return x_83; -} +lean_object* x_39; lean_object* x_40; +lean_dec(x_4); +x_39 = lean_box(0); +x_40 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1(x_5, x_6, x_2, x_1, x_20, x_25, x_39, x_9, x_10, x_11, x_12, x_13, x_14, x_28); +lean_dec(x_20); +return x_40; } } else { -lean_object* x_84; lean_object* x_85; lean_object* x_86; size_t x_87; size_t x_88; size_t x_89; lean_object* x_90; uint8_t x_91; -x_84 = lean_ctor_get(x_32, 0); -x_85 = lean_ctor_get(x_32, 1); -lean_inc(x_85); -lean_inc(x_84); -lean_dec(x_32); -x_86 = lean_array_get_size(x_85); -x_87 = lean_usize_of_nat(x_86); -lean_dec(x_86); -x_88 = lean_usize_sub(x_87, x_25); -x_89 = lean_usize_land(x_23, x_88); -x_90 = lean_array_uget(x_85, x_89); -x_91 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_CollectLevelMVars_visitExpr___spec__1(x_1, x_90); -if (x_91 == 0) -{ -lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; uint8_t x_102; -x_92 = lean_unsigned_to_nat(1u); -x_93 = lean_nat_add(x_84, x_92); -lean_dec(x_84); -x_94 = lean_box(0); -x_95 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_95, 0, x_1); -lean_ctor_set(x_95, 1, x_94); -lean_ctor_set(x_95, 2, x_90); -x_96 = lean_array_uset(x_85, x_89, x_95); -x_97 = lean_unsigned_to_nat(4u); -x_98 = lean_nat_mul(x_93, x_97); -x_99 = lean_unsigned_to_nat(3u); -x_100 = lean_nat_div(x_98, x_99); -lean_dec(x_98); -x_101 = lean_array_get_size(x_96); -x_102 = lean_nat_dec_le(x_100, x_101); -lean_dec(x_101); -lean_dec(x_100); -if (x_102 == 0) +uint8_t x_41; +lean_dec(x_25); +lean_dec(x_20); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +x_41 = !lean_is_exclusive(x_26); +if (x_41 == 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; lean_object* x_109; lean_object* x_110; -x_103 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_CollectLevelMVars_visitExpr___spec__2(x_96); -x_104 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_104, 0, x_93); -lean_ctor_set(x_104, 1, x_103); -lean_ctor_set(x_31, 1, x_104); -x_105 = lean_st_ref_set(x_2, x_31, x_33); -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 = 0; -x_109 = lean_box(x_108); -if (lean_is_scalar(x_107)) { - x_110 = lean_alloc_ctor(0, 2, 0); -} else { - x_110 = x_107; -} -lean_ctor_set(x_110, 0, x_109); -lean_ctor_set(x_110, 1, x_106); -return x_110; +return x_26; } else { -lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; uint8_t x_115; lean_object* x_116; lean_object* x_117; -x_111 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_111, 0, x_93); -lean_ctor_set(x_111, 1, x_96); -lean_ctor_set(x_31, 1, x_111); -x_112 = lean_st_ref_set(x_2, x_31, x_33); -x_113 = lean_ctor_get(x_112, 1); -lean_inc(x_113); -if (lean_is_exclusive(x_112)) { - lean_ctor_release(x_112, 0); - lean_ctor_release(x_112, 1); - x_114 = x_112; -} else { - lean_dec_ref(x_112); - x_114 = lean_box(0); -} -x_115 = 0; -x_116 = lean_box(x_115); -if (lean_is_scalar(x_114)) { - x_117 = lean_alloc_ctor(0, 2, 0); -} else { - x_117 = x_114; +lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_42 = lean_ctor_get(x_26, 0); +x_43 = lean_ctor_get(x_26, 1); +lean_inc(x_43); +lean_inc(x_42); +lean_dec(x_26); +x_44 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_44, 0, x_42); +lean_ctor_set(x_44, 1, x_43); +return x_44; } -lean_ctor_set(x_117, 0, x_116); -lean_ctor_set(x_117, 1, x_113); -return x_117; } } else { -lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; uint8_t x_122; lean_object* x_123; lean_object* x_124; -lean_dec(x_90); -lean_dec(x_1); -x_118 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_118, 0, x_84); -lean_ctor_set(x_118, 1, x_85); -lean_ctor_set(x_31, 1, x_118); -x_119 = lean_st_ref_set(x_2, x_31, x_33); -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 = 0; -x_123 = lean_box(x_122); -if (lean_is_scalar(x_121)) { - x_124 = lean_alloc_ctor(0, 2, 0); -} else { - x_124 = x_121; -} -lean_ctor_set(x_124, 0, x_123); -lean_ctor_set(x_124, 1, x_120); -return x_124; +lean_object* x_45; lean_object* x_46; +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_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_45 = lean_box(0); +x_46 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_46, 0, x_45); +lean_ctor_set(x_46, 1, x_15); +return x_46; } } } -else +case 5: { -lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; size_t x_130; size_t x_131; size_t x_132; lean_object* x_133; uint8_t x_134; -x_125 = lean_ctor_get(x_31, 0); -lean_inc(x_125); -lean_dec(x_31); -x_126 = lean_ctor_get(x_32, 0); -lean_inc(x_126); -x_127 = lean_ctor_get(x_32, 1); -lean_inc(x_127); -if (lean_is_exclusive(x_32)) { - lean_ctor_release(x_32, 0); - lean_ctor_release(x_32, 1); - x_128 = x_32; -} else { - lean_dec_ref(x_32); - x_128 = lean_box(0); -} -x_129 = lean_array_get_size(x_127); -x_130 = lean_usize_of_nat(x_129); -lean_dec(x_129); -x_131 = lean_usize_sub(x_130, x_25); -x_132 = lean_usize_land(x_23, x_131); -x_133 = lean_array_uget(x_127, x_132); -x_134 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_CollectLevelMVars_visitExpr___spec__1(x_1, x_133); -if (x_134 == 0) +switch (lean_obj_tag(x_8)) { +case 0: { -lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; uint8_t x_145; -x_135 = lean_unsigned_to_nat(1u); -x_136 = lean_nat_add(x_126, x_135); -lean_dec(x_126); -x_137 = lean_box(0); -x_138 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_138, 0, x_1); -lean_ctor_set(x_138, 1, x_137); -lean_ctor_set(x_138, 2, x_133); -x_139 = lean_array_uset(x_127, x_132, x_138); -x_140 = lean_unsigned_to_nat(4u); -x_141 = lean_nat_mul(x_136, x_140); -x_142 = lean_unsigned_to_nat(3u); -x_143 = lean_nat_div(x_141, x_142); -lean_dec(x_141); -x_144 = lean_array_get_size(x_139); -x_145 = lean_nat_dec_le(x_143, x_144); -lean_dec(x_144); -lean_dec(x_143); -if (x_145 == 0) +lean_object* x_47; lean_object* x_48; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_47 = lean_ctor_get(x_7, 0); +lean_inc(x_47); +lean_dec(x_7); +x_48 = l_Lean_assignLevelMVar___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___spec__1(x_47, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +return x_48; +} +case 4: { -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; lean_object* x_153; lean_object* x_154; -x_146 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_CollectLevelMVars_visitExpr___spec__2(x_139); -if (lean_is_scalar(x_128)) { - x_147 = lean_alloc_ctor(0, 2, 0); -} else { - x_147 = x_128; +lean_object* x_49; lean_object* x_50; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_49 = lean_ctor_get(x_7, 0); +lean_inc(x_49); +lean_dec(x_7); +x_50 = l_Lean_assignLevelMVar___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___spec__1(x_49, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +return x_50; } -lean_ctor_set(x_147, 0, x_136); -lean_ctor_set(x_147, 1, x_146); -x_148 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_148, 0, x_125); -lean_ctor_set(x_148, 1, x_147); -x_149 = lean_st_ref_set(x_2, x_148, x_33); -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; -} else { - lean_dec_ref(x_149); - x_151 = lean_box(0); +default: +{ +uint8_t x_51; +lean_dec(x_8); +lean_dec(x_7); +x_51 = l_Lean_Level_geq(x_2, x_6); +if (x_51 == 0) +{ +lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; +x_52 = lean_ctor_get(x_3, 0); +lean_inc(x_52); +lean_dec(x_3); +lean_inc(x_52); +x_53 = l_Lean_MessageData_ofName(x_52); +x_54 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___closed__2; +x_55 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_55, 0, x_54); +lean_ctor_set(x_55, 1, x_53); +x_56 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___closed__4; +x_57 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_57, 0, x_55); +lean_ctor_set(x_57, 1, x_56); +lean_inc(x_11); +x_58 = l_Lean_Meta_getFVarLocalDecl(x_4, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_58) == 0) +{ +lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; +x_59 = lean_ctor_get(x_58, 0); +lean_inc(x_59); +x_60 = lean_ctor_get(x_58, 1); +lean_inc(x_60); +lean_dec(x_58); +x_61 = l_Lean_LocalDecl_userName(x_59); +lean_dec(x_59); +x_62 = l_Lean_Name_hasMacroScopes(x_61); +lean_dec(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; +x_63 = l_Lean_MessageData_ofExpr(x_4); +x_64 = l_Lean_Elab_Command_accLevelAtCtor___closed__8; +x_65 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_65, 0, x_64); +lean_ctor_set(x_65, 1, x_63); +x_66 = l_Lean_Elab_Command_accLevelAtCtor___closed__10; +x_67 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_67, 0, x_65); +lean_ctor_set(x_67, 1, x_66); +x_68 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_68, 0, x_57); +lean_ctor_set(x_68, 1, x_67); +x_69 = lean_box(0); +x_70 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1(x_5, x_6, x_2, x_1, x_52, x_68, x_69, x_9, x_10, x_11, x_12, x_13, x_14, x_60); +lean_dec(x_52); +return x_70; } -x_152 = 0; -x_153 = lean_box(x_152); -if (lean_is_scalar(x_151)) { - x_154 = lean_alloc_ctor(0, 2, 0); -} else { - x_154 = x_151; +else +{ +lean_object* x_71; lean_object* x_72; +lean_dec(x_4); +x_71 = lean_box(0); +x_72 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1(x_5, x_6, x_2, x_1, x_52, x_57, x_71, x_9, x_10, x_11, x_12, x_13, x_14, x_60); +lean_dec(x_52); +return x_72; } -lean_ctor_set(x_154, 0, x_153); -lean_ctor_set(x_154, 1, x_150); -return x_154; } 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; lean_object* x_161; lean_object* x_162; -if (lean_is_scalar(x_128)) { - x_155 = lean_alloc_ctor(0, 2, 0); -} else { - x_155 = x_128; -} -lean_ctor_set(x_155, 0, x_136); -lean_ctor_set(x_155, 1, x_139); -x_156 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_156, 0, x_125); -lean_ctor_set(x_156, 1, x_155); -x_157 = lean_st_ref_set(x_2, x_156, x_33); -x_158 = lean_ctor_get(x_157, 1); -lean_inc(x_158); -if (lean_is_exclusive(x_157)) { - lean_ctor_release(x_157, 0); - lean_ctor_release(x_157, 1); - x_159 = x_157; -} else { - lean_dec_ref(x_157); - x_159 = lean_box(0); +uint8_t x_73; +lean_dec(x_57); +lean_dec(x_52); +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_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +x_73 = !lean_is_exclusive(x_58); +if (x_73 == 0) +{ +return x_58; } -x_160 = 0; -x_161 = lean_box(x_160); -if (lean_is_scalar(x_159)) { - x_162 = lean_alloc_ctor(0, 2, 0); -} else { - x_162 = x_159; +else +{ +lean_object* x_74; lean_object* x_75; lean_object* x_76; +x_74 = lean_ctor_get(x_58, 0); +x_75 = lean_ctor_get(x_58, 1); +lean_inc(x_75); +lean_inc(x_74); +lean_dec(x_58); +x_76 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_76, 0, x_74); +lean_ctor_set(x_76, 1, x_75); +return x_76; } -lean_ctor_set(x_162, 0, x_161); -lean_ctor_set(x_162, 1, x_158); -return x_162; } } else { -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_dec(x_133); -lean_dec(x_1); -if (lean_is_scalar(x_128)) { - x_163 = lean_alloc_ctor(0, 2, 0); -} else { - x_163 = x_128; -} -lean_ctor_set(x_163, 0, x_126); -lean_ctor_set(x_163, 1, x_127); -x_164 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_164, 0, x_125); -lean_ctor_set(x_164, 1, x_163); -x_165 = lean_st_ref_set(x_2, x_164, x_33); -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; -} else { - lean_dec_ref(x_165); - x_167 = lean_box(0); +lean_object* x_77; lean_object* x_78; +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_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_77 = lean_box(0); +x_78 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_78, 0, x_77); +lean_ctor_set(x_78, 1, x_15); +return x_78; } -x_168 = 0; -x_169 = lean_box(x_168); -if (lean_is_scalar(x_167)) { - x_170 = lean_alloc_ctor(0, 2, 0); -} else { - x_170 = x_167; } -lean_ctor_set(x_170, 0, x_169); -lean_ctor_set(x_170, 1, x_166); -return x_170; } } +default: +{ +uint8_t x_79; +lean_dec(x_8); +lean_dec(x_7); +x_79 = l_Lean_Level_geq(x_2, x_6); +if (x_79 == 0) +{ +lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; +x_80 = lean_ctor_get(x_3, 0); +lean_inc(x_80); +lean_dec(x_3); +lean_inc(x_80); +x_81 = l_Lean_MessageData_ofName(x_80); +x_82 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___closed__2; +x_83 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_83, 0, x_82); +lean_ctor_set(x_83, 1, x_81); +x_84 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___closed__4; +x_85 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_85, 0, x_83); +lean_ctor_set(x_85, 1, x_84); +lean_inc(x_11); +x_86 = l_Lean_Meta_getFVarLocalDecl(x_4, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_86) == 0) +{ +lean_object* x_87; lean_object* x_88; lean_object* x_89; uint8_t 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 = l_Lean_LocalDecl_userName(x_87); +lean_dec(x_87); +x_90 = l_Lean_Name_hasMacroScopes(x_89); +lean_dec(x_89); +if (x_90 == 0) +{ +lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; +x_91 = l_Lean_MessageData_ofExpr(x_4); +x_92 = l_Lean_Elab_Command_accLevelAtCtor___closed__8; +x_93 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_93, 0, x_92); +lean_ctor_set(x_93, 1, x_91); +x_94 = l_Lean_Elab_Command_accLevelAtCtor___closed__10; +x_95 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_95, 0, x_93); +lean_ctor_set(x_95, 1, x_94); +x_96 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_96, 0, x_85); +lean_ctor_set(x_96, 1, x_95); +x_97 = lean_box(0); +x_98 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1(x_5, x_6, x_2, x_1, x_80, x_96, x_97, x_9, x_10, x_11, x_12, x_13, x_14, x_88); +lean_dec(x_80); +return x_98; } else { -uint8_t x_171; lean_object* x_172; -lean_dec(x_1); -x_171 = 1; -x_172 = lean_box(x_171); -lean_ctor_set(x_8, 0, x_172); -return x_8; +lean_object* x_99; lean_object* x_100; +lean_dec(x_4); +x_99 = lean_box(0); +x_100 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1(x_5, x_6, x_2, x_1, x_80, x_85, x_99, x_9, x_10, x_11, x_12, x_13, x_14, x_88); +lean_dec(x_80); +return x_100; } } else { -lean_object* x_173; lean_object* x_174; lean_object* x_175; uint64_t x_176; uint64_t x_177; uint64_t x_178; uint64_t x_179; uint64_t x_180; uint64_t x_181; uint64_t x_182; size_t x_183; size_t x_184; size_t x_185; size_t x_186; size_t x_187; lean_object* x_188; uint8_t x_189; -x_173 = lean_ctor_get(x_8, 1); -lean_inc(x_173); -lean_dec(x_8); -x_174 = lean_ctor_get(x_10, 1); -lean_inc(x_174); +uint8_t x_101; +lean_dec(x_85); +lean_dec(x_80); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); lean_dec(x_10); -x_175 = lean_array_get_size(x_174); -x_176 = l_Lean_Expr_hash(x_1); -x_177 = 32; -x_178 = lean_uint64_shift_right(x_176, x_177); -x_179 = lean_uint64_xor(x_176, x_178); -x_180 = 16; -x_181 = lean_uint64_shift_right(x_179, x_180); -x_182 = lean_uint64_xor(x_179, x_181); -x_183 = lean_uint64_to_usize(x_182); -x_184 = lean_usize_of_nat(x_175); -lean_dec(x_175); -x_185 = 1; -x_186 = lean_usize_sub(x_184, x_185); -x_187 = lean_usize_land(x_183, x_186); -x_188 = lean_array_uget(x_174, x_187); -lean_dec(x_174); -x_189 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_CollectLevelMVars_visitExpr___spec__1(x_1, x_188); -lean_dec(x_188); -if (x_189 == 0) +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +x_101 = !lean_is_exclusive(x_86); +if (x_101 == 0) { -lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; size_t x_200; size_t x_201; size_t x_202; lean_object* x_203; uint8_t x_204; -x_190 = lean_st_ref_take(x_2, x_173); -x_191 = lean_ctor_get(x_190, 0); -lean_inc(x_191); -x_192 = lean_ctor_get(x_191, 1); -lean_inc(x_192); -x_193 = lean_ctor_get(x_190, 1); -lean_inc(x_193); -lean_dec(x_190); -x_194 = lean_ctor_get(x_191, 0); -lean_inc(x_194); -if (lean_is_exclusive(x_191)) { - lean_ctor_release(x_191, 0); - lean_ctor_release(x_191, 1); - x_195 = x_191; -} else { - lean_dec_ref(x_191); - x_195 = lean_box(0); -} -x_196 = lean_ctor_get(x_192, 0); -lean_inc(x_196); -x_197 = lean_ctor_get(x_192, 1); -lean_inc(x_197); -if (lean_is_exclusive(x_192)) { - lean_ctor_release(x_192, 0); - lean_ctor_release(x_192, 1); - x_198 = x_192; -} else { - lean_dec_ref(x_192); - x_198 = lean_box(0); +return x_86; } -x_199 = lean_array_get_size(x_197); -x_200 = lean_usize_of_nat(x_199); -lean_dec(x_199); -x_201 = lean_usize_sub(x_200, x_185); -x_202 = lean_usize_land(x_183, x_201); -x_203 = lean_array_uget(x_197, x_202); -x_204 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_CollectLevelMVars_visitExpr___spec__1(x_1, x_203); -if (x_204 == 0) +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; uint8_t x_215; -x_205 = lean_unsigned_to_nat(1u); -x_206 = lean_nat_add(x_196, x_205); -lean_dec(x_196); -x_207 = lean_box(0); -x_208 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_208, 0, x_1); -lean_ctor_set(x_208, 1, x_207); -lean_ctor_set(x_208, 2, x_203); -x_209 = lean_array_uset(x_197, x_202, x_208); -x_210 = lean_unsigned_to_nat(4u); -x_211 = lean_nat_mul(x_206, x_210); -x_212 = lean_unsigned_to_nat(3u); -x_213 = lean_nat_div(x_211, x_212); -lean_dec(x_211); -x_214 = lean_array_get_size(x_209); -x_215 = lean_nat_dec_le(x_213, x_214); -lean_dec(x_214); -lean_dec(x_213); -if (x_215 == 0) +lean_object* x_102; lean_object* x_103; lean_object* x_104; +x_102 = lean_ctor_get(x_86, 0); +x_103 = lean_ctor_get(x_86, 1); +lean_inc(x_103); +lean_inc(x_102); +lean_dec(x_86); +x_104 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_104, 0, x_102); +lean_ctor_set(x_104, 1, x_103); +return x_104; +} +} +} +else { -lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; uint8_t x_222; lean_object* x_223; lean_object* x_224; -x_216 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_CollectLevelMVars_visitExpr___spec__2(x_209); -if (lean_is_scalar(x_198)) { - x_217 = lean_alloc_ctor(0, 2, 0); -} else { - x_217 = x_198; +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_10); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_105 = lean_box(0); +x_106 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_106, 0, x_105); +lean_ctor_set(x_106, 1, x_15); +return x_106; } -lean_ctor_set(x_217, 0, x_206); -lean_ctor_set(x_217, 1, x_216); -if (lean_is_scalar(x_195)) { - x_218 = lean_alloc_ctor(0, 2, 0); -} else { - x_218 = x_195; } -lean_ctor_set(x_218, 0, x_194); -lean_ctor_set(x_218, 1, x_217); -x_219 = lean_st_ref_set(x_2, x_218, x_193); -x_220 = lean_ctor_get(x_219, 1); -lean_inc(x_220); -if (lean_is_exclusive(x_219)) { - lean_ctor_release(x_219, 0); - lean_ctor_release(x_219, 1); - x_221 = x_219; -} else { - lean_dec_ref(x_219); - x_221 = lean_box(0); } -x_222 = 0; -x_223 = lean_box(x_222); -if (lean_is_scalar(x_221)) { - x_224 = lean_alloc_ctor(0, 2, 0); -} else { - x_224 = x_221; } -lean_ctor_set(x_224, 0, x_223); -lean_ctor_set(x_224, 1, x_220); -return x_224; } -else +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: { -lean_object* x_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; -if (lean_is_scalar(x_198)) { - x_225 = lean_alloc_ctor(0, 2, 0); -} else { - x_225 = x_198; -} -lean_ctor_set(x_225, 0, x_206); -lean_ctor_set(x_225, 1, x_209); -if (lean_is_scalar(x_195)) { - x_226 = lean_alloc_ctor(0, 2, 0); -} else { - x_226 = x_195; -} -lean_ctor_set(x_226, 0, x_194); -lean_ctor_set(x_226, 1, x_225); -x_227 = lean_st_ref_set(x_2, x_226, x_193); -x_228 = lean_ctor_get(x_227, 1); -lean_inc(x_228); -if (lean_is_exclusive(x_227)) { - lean_ctor_release(x_227, 0); - lean_ctor_release(x_227, 1); - x_229 = x_227; -} else { - lean_dec_ref(x_227); - x_229 = lean_box(0); -} -x_230 = 0; -x_231 = lean_box(x_230); -if (lean_is_scalar(x_229)) { - x_232 = lean_alloc_ctor(0, 2, 0); -} else { - x_232 = x_229; -} -lean_ctor_set(x_232, 0, x_231); -lean_ctor_set(x_232, 1, x_228); -return x_232; +size_t x_15; size_t x_16; lean_object* x_17; +x_15 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_16 = lean_unbox_usize(x_6); +lean_dec(x_6); +x_17 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___spec__2(x_1, x_2, x_3, x_4, x_15, x_16, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_4); +lean_dec(x_1); +return x_17; } } -else +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___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) { +_start: { -lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; uint8_t x_238; lean_object* x_239; lean_object* x_240; -lean_dec(x_203); +size_t x_15; size_t x_16; lean_object* x_17; +x_15 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_16 = lean_unbox_usize(x_6); +lean_dec(x_6); +x_17 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___spec__3(x_1, x_2, x_3, x_4, x_15, x_16, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_4); lean_dec(x_1); -if (lean_is_scalar(x_198)) { - x_233 = lean_alloc_ctor(0, 2, 0); -} else { - x_233 = x_198; -} -lean_ctor_set(x_233, 0, x_196); -lean_ctor_set(x_233, 1, x_197); -if (lean_is_scalar(x_195)) { - x_234 = lean_alloc_ctor(0, 2, 0); -} else { - x_234 = x_195; -} -lean_ctor_set(x_234, 0, x_194); -lean_ctor_set(x_234, 1, x_233); -x_235 = lean_st_ref_set(x_2, x_234, x_193); -x_236 = lean_ctor_get(x_235, 1); -lean_inc(x_236); -if (lean_is_exclusive(x_235)) { - lean_ctor_release(x_235, 0); - lean_ctor_release(x_235, 1); - x_237 = x_235; -} else { - lean_dec_ref(x_235); - x_237 = lean_box(0); +return x_17; } -x_238 = 0; -x_239 = lean_box(x_238); -if (lean_is_scalar(x_237)) { - x_240 = lean_alloc_ctor(0, 2, 0); -} else { - x_240 = x_237; } -lean_ctor_set(x_240, 0, x_239); -lean_ctor_set(x_240, 1, x_236); -return x_240; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_withCtorRef___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l_Lean_Elab_Command_withCtorRef___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_2); +return x_10; } } -else +LEAN_EXPORT lean_object* l_Lean_Elab_Command_withCtorRef___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: { -uint8_t x_241; lean_object* x_242; lean_object* x_243; +lean_object* x_11; +x_11 = l_Lean_Elab_Command_withCtorRef___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___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_2); lean_dec(x_1); -x_241 = 1; -x_242 = lean_box(x_241); -x_243 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_243, 0, x_242); -lean_ctor_set(x_243, 1, x_173); -return x_243; +return x_11; } } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; +x_15 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___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_7); +lean_dec(x_5); +lean_dec(x_4); +return x_15; } } -LEAN_EXPORT lean_object* l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { -switch (lean_obj_tag(x_1)) { -case 5: -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_12 = lean_ctor_get(x_1, 0); -lean_inc(x_12); -x_13 = lean_ctor_get(x_1, 1); -lean_inc(x_13); +lean_object* x_16; +x_16 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check(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_1); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_3); -lean_inc(x_2); -x_14 = l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6(x_2, x_3, x_4, x_12, 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; -x_15 = lean_ctor_get(x_14, 1); -lean_inc(x_15); -lean_dec(x_14); -x_16 = l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6(x_2, x_3, x_4, x_13, x_6, x_7, x_8, x_9, x_10, x_15); return x_16; } -else +} +LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: { -uint8_t x_17; +uint8_t x_15; +x_15 = lean_usize_dec_lt(x_6, x_5); +if (x_15 == 0) +{ +lean_object* x_16; lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_7); lean_dec(x_3); lean_dec(x_2); -x_17 = !lean_is_exclusive(x_14); -if (x_17 == 0) -{ -return x_14; +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_7); +lean_ctor_set(x_16, 1, x_14); +return x_16; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_14, 0); -x_19 = lean_ctor_get(x_14, 1); -lean_inc(x_19); +lean_object* x_17; lean_object* x_18; lean_object* x_19; +lean_dec(x_7); +x_17 = lean_ctor_get(x_4, 0); +x_18 = lean_array_uget(x_17, x_6); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); lean_inc(x_18); -lean_dec(x_14); -x_20 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_20, 0, x_18); -lean_ctor_set(x_20, 1, x_19); -return x_20; -} -} -} -case 6: +x_19 = lean_infer_type(x_18, x_10, x_11, x_12, x_13, x_14); +if (lean_obj_tag(x_19) == 0) { -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_1, 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); +x_21 = lean_ctor_get(x_19, 1); lean_inc(x_21); -x_22 = lean_ctor_get(x_1, 2); -lean_inc(x_22); -lean_dec(x_1); +lean_dec(x_19); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_3); -lean_inc(x_2); -x_23 = l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6(x_2, x_3, x_4, x_21, x_6, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_23) == 0) +lean_inc(x_20); +x_22 = l_Lean_Meta_getLevel(x_20, x_10, x_11, x_12, x_13, x_21); +if (lean_obj_tag(x_22) == 0) { -lean_object* x_24; lean_object* x_25; -x_24 = lean_ctor_get(x_23, 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; +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_23); -x_25 = l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6(x_2, x_3, x_4, x_22, x_6, x_7, x_8, x_9, x_10, x_24); -return x_25; -} -else -{ -uint8_t x_26; lean_dec(x_22); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -x_26 = !lean_is_exclusive(x_23); -if (x_26 == 0) -{ -return x_23; -} -else -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_23, 0); -x_28 = lean_ctor_get(x_23, 1); -lean_inc(x_28); +x_25 = l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_shouldInferResultUniverse___spec__1(x_23, x_8, x_9, x_10, x_11, x_12, x_13, 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_23); -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; -} -} -} -case 7: -{ -lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_30 = lean_ctor_get(x_1, 1); -lean_inc(x_30); -x_31 = lean_ctor_get(x_1, 2); -lean_inc(x_31); -lean_dec(x_1); +lean_dec(x_25); +x_28 = l_Lean_Level_normalize(x_26); +lean_dec(x_26); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -lean_inc(x_7); +lean_inc(x_28); lean_inc(x_3); -lean_inc(x_2); -x_32 = l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6(x_2, x_3, x_4, x_30, x_6, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_32) == 0) +lean_inc_n(x_2, 2); +x_29 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check(x_1, x_2, x_3, x_18, x_20, x_28, x_28, x_2, x_8, x_9, x_10, x_11, x_12, x_13, x_27); +if (lean_obj_tag(x_29) == 0) { -lean_object* x_33; lean_object* x_34; -x_33 = lean_ctor_get(x_32, 1); -lean_inc(x_33); -lean_dec(x_32); -x_34 = l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6(x_2, x_3, x_4, x_31, x_6, x_7, x_8, x_9, x_10, x_33); -return x_34; +lean_object* x_30; size_t x_31; size_t x_32; lean_object* x_33; +x_30 = lean_ctor_get(x_29, 1); +lean_inc(x_30); +lean_dec(x_29); +x_31 = 1; +x_32 = lean_usize_add(x_6, x_31); +x_33 = lean_box(0); +x_6 = x_32; +x_7 = x_33; +x_14 = x_30; +goto _start; } else { uint8_t x_35; -lean_dec(x_31); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_7); lean_dec(x_3); lean_dec(x_2); -x_35 = !lean_is_exclusive(x_32); +x_35 = !lean_is_exclusive(x_29); if (x_35 == 0) { -return x_32; +return x_29; } else { lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_32, 0); -x_37 = lean_ctor_get(x_32, 1); +x_36 = lean_ctor_get(x_29, 0); +x_37 = lean_ctor_get(x_29, 1); lean_inc(x_37); lean_inc(x_36); -lean_dec(x_32); +lean_dec(x_29); x_38 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_38, 0, x_36); lean_ctor_set(x_38, 1, x_37); @@ -23601,774 +24111,850 @@ return x_38; } } } -case 8: -{ -lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_39 = lean_ctor_get(x_1, 1); -lean_inc(x_39); -x_40 = lean_ctor_get(x_1, 2); -lean_inc(x_40); -x_41 = lean_ctor_get(x_1, 3); -lean_inc(x_41); -lean_dec(x_1); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_3); -lean_inc(x_2); -x_42 = l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6(x_2, x_3, x_4, x_39, x_6, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_42) == 0) -{ -lean_object* x_43; lean_object* x_44; -x_43 = lean_ctor_get(x_42, 1); -lean_inc(x_43); -lean_dec(x_42); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_3); -lean_inc(x_2); -x_44 = l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6(x_2, x_3, x_4, x_40, x_6, x_7, x_8, x_9, x_10, x_43); -if (lean_obj_tag(x_44) == 0) -{ -lean_object* x_45; lean_object* x_46; -x_45 = lean_ctor_get(x_44, 1); -lean_inc(x_45); -lean_dec(x_44); -x_46 = l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6(x_2, x_3, x_4, x_41, x_6, x_7, x_8, x_9, x_10, x_45); -return x_46; -} else { -uint8_t x_47; -lean_dec(x_41); +uint8_t x_39; +lean_dec(x_20); +lean_dec(x_18); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_7); lean_dec(x_3); lean_dec(x_2); -x_47 = !lean_is_exclusive(x_44); -if (x_47 == 0) +x_39 = !lean_is_exclusive(x_22); +if (x_39 == 0) { -return x_44; +return x_22; } 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_40; lean_object* x_41; lean_object* x_42; +x_40 = lean_ctor_get(x_22, 0); +x_41 = lean_ctor_get(x_22, 1); +lean_inc(x_41); +lean_inc(x_40); +lean_dec(x_22); +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_51; -lean_dec(x_41); -lean_dec(x_40); +uint8_t x_43; +lean_dec(x_18); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_7); lean_dec(x_3); lean_dec(x_2); -x_51 = !lean_is_exclusive(x_42); -if (x_51 == 0) +x_43 = !lean_is_exclusive(x_19); +if (x_43 == 0) { -return x_42; +return x_19; } else { -lean_object* x_52; lean_object* x_53; lean_object* x_54; -x_52 = lean_ctor_get(x_42, 0); -x_53 = lean_ctor_get(x_42, 1); -lean_inc(x_53); -lean_inc(x_52); -lean_dec(x_42); -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_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; } } } -case 10: +} +} +LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses___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_55; lean_object* x_56; -x_55 = lean_ctor_get(x_1, 1); -lean_inc(x_55); -lean_dec(x_1); -x_56 = l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6(x_2, x_3, x_4, x_55, x_6, x_7, x_8, x_9, x_10, x_11); -return x_56; +lean_object* x_14; lean_object* x_15; lean_object* x_16; size_t x_17; lean_object* x_18; size_t x_19; lean_object* x_20; lean_object* x_21; +x_14 = lean_array_get_size(x_5); +x_15 = l_Array_toSubarray___rarg(x_5, x_1, x_14); +x_16 = lean_ctor_get(x_15, 2); +lean_inc(x_16); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = lean_ctor_get(x_15, 1); +lean_inc(x_18); +x_19 = lean_usize_of_nat(x_18); +lean_dec(x_18); +x_20 = lean_box(0); +x_21 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses___spec__1(x_2, x_3, x_4, x_15, x_17, x_19, x_20, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_15); +if (lean_obj_tag(x_21) == 0) +{ +uint8_t x_22; +x_22 = !lean_is_exclusive(x_21); +if (x_22 == 0) +{ +lean_object* x_23; +x_23 = lean_ctor_get(x_21, 0); +lean_dec(x_23); +lean_ctor_set(x_21, 0, x_20); +return x_21; } -case 11: +else { -lean_object* x_57; lean_object* x_58; -x_57 = lean_ctor_get(x_1, 2); -lean_inc(x_57); -lean_dec(x_1); -x_58 = l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6(x_2, x_3, x_4, x_57, x_6, x_7, x_8, x_9, x_10, x_11); -return x_58; +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_21, 1); +lean_inc(x_24); +lean_dec(x_21); +x_25 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_25, 0, x_20); +lean_ctor_set(x_25, 1, x_24); +return x_25; } -default: +} +else { -lean_object* x_59; lean_object* x_60; +uint8_t x_26; +x_26 = !lean_is_exclusive(x_21); +if (x_26 == 0) +{ +return x_21; +} +else +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_21, 0); +x_28 = lean_ctor_get(x_21, 1); +lean_inc(x_28); +lean_inc(x_27); +lean_dec(x_21); +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_27); +lean_ctor_set(x_29, 1, x_28); +return x_29; +} +} +} +} +LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +if (lean_obj_tag(x_4) == 0) +{ +lean_object* x_12; lean_object* x_13; lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); lean_dec(x_3); lean_dec(x_2); 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_11); -return x_60; -} -} -} +x_12 = lean_box(0); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_11); +return x_13; } -LEAN_EXPORT lean_object* l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; lean_object* x_12; uint8_t x_13; -lean_inc(x_4); -x_11 = l_Lean_ForEachExprWhere_visited___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__7(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_unbox(x_12); -lean_dec(x_12); -if (x_13 == 0) +else { -lean_object* x_14; lean_object* x_15; uint8_t x_16; -x_14 = lean_ctor_get(x_11, 1); +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_14 = lean_ctor_get(x_4, 0); lean_inc(x_14); -lean_dec(x_11); +x_15 = lean_ctor_get(x_4, 1); +lean_inc(x_15); +lean_dec(x_4); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_inc(x_3); lean_inc(x_1); -lean_inc(x_4); -x_15 = lean_apply_1(x_1, x_4); -x_16 = lean_unbox(x_15); -lean_dec(x_15); -if (x_16 == 0) -{ -lean_object* x_17; lean_object* x_18; -x_17 = lean_box(0); -x_18 = l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6___lambda__1(x_4, x_1, x_2, x_3, x_17, x_5, x_6, x_7, x_8, x_9, x_14); -return x_18; -} -else -{ -lean_object* x_19; lean_object* x_20; uint8_t x_21; -lean_inc(x_4); -x_19 = l_Lean_ForEachExprWhere_checked___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__8(x_4, x_5, x_6, x_7, x_8, x_9, x_14); -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); -x_21 = lean_unbox(x_20); -lean_dec(x_20); -if (x_21 == 0) -{ -lean_object* x_22; lean_object* x_23; -x_22 = lean_ctor_get(x_19, 1); -lean_inc(x_22); -lean_dec(x_19); lean_inc(x_2); +x_17 = lean_alloc_closure((void*)(l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses___spec__2___lambda__1___boxed), 13, 4); +lean_closure_set(x_17, 0, x_2); +lean_closure_set(x_17, 1, x_1); +lean_closure_set(x_17, 2, x_3); +lean_closure_set(x_17, 3, x_14); +x_18 = 0; +lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -lean_inc(x_4); -x_23 = lean_apply_6(x_2, x_4, x_6, x_7, x_8, x_9, x_22); -if (lean_obj_tag(x_23) == 0) -{ -if (x_3 == 0) +lean_inc(x_5); +x_19 = l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___spec__1___rarg(x_16, x_17, x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_19) == 0) { -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_23, 1); -lean_inc(x_24); -lean_dec(x_23); -x_25 = lean_box(0); -x_26 = l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6___lambda__1(x_4, x_1, x_2, x_3, x_25, x_5, x_6, x_7, x_8, x_9, x_24); -return x_26; +lean_object* x_20; +x_20 = lean_ctor_get(x_19, 1); +lean_inc(x_20); +lean_dec(x_19); +x_4 = x_15; +x_11 = x_20; +goto _start; } else { -uint8_t x_27; +uint8_t x_22; +lean_dec(x_15); +lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_4); +lean_dec(x_5); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_27 = !lean_is_exclusive(x_23); -if (x_27 == 0) +x_22 = !lean_is_exclusive(x_19); +if (x_22 == 0) { -lean_object* x_28; lean_object* x_29; -x_28 = lean_ctor_get(x_23, 0); -lean_dec(x_28); -x_29 = lean_box(0); -lean_ctor_set(x_23, 0, x_29); -return x_23; +return x_19; } else { -lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_30 = lean_ctor_get(x_23, 1); -lean_inc(x_30); -lean_dec(x_23); -x_31 = lean_box(0); -x_32 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_32, 0, x_31); -lean_ctor_set(x_32, 1, x_30); -return x_32; +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_19, 0); +x_24 = lean_ctor_get(x_19, 1); +lean_inc(x_24); +lean_inc(x_23); +lean_dec(x_19); +x_25 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +return x_25; } } } -else +} +} +LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: { -uint8_t x_33; +if (lean_obj_tag(x_4) == 0) +{ +lean_object* x_12; lean_object* x_13; +lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_4); +lean_dec(x_5); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_33 = !lean_is_exclusive(x_23); -if (x_33 == 0) -{ -return x_23; +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_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_23, 0); -x_35 = lean_ctor_get(x_23, 1); -lean_inc(x_35); -lean_inc(x_34); -lean_dec(x_23); -x_36 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_36, 0, x_34); -lean_ctor_set(x_36, 1, x_35); -return x_36; -} -} -} -else +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +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); +x_16 = lean_ctor_get(x_14, 2); +lean_inc(x_16); +lean_dec(x_14); +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); +lean_inc(x_1); +x_17 = l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses___spec__2(x_1, x_2, x_3, x_16, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_17) == 0) { -lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_37 = lean_ctor_get(x_19, 1); -lean_inc(x_37); -lean_dec(x_19); -x_38 = lean_box(0); -x_39 = l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6___lambda__1(x_4, x_1, x_2, x_3, x_38, x_5, x_6, x_7, x_8, x_9, x_37); -return x_39; -} -} +lean_object* x_18; +x_18 = lean_ctor_get(x_17, 1); +lean_inc(x_18); +lean_dec(x_17); +x_4 = x_15; +x_11 = x_18; +goto _start; } else { -uint8_t x_40; +uint8_t x_20; +lean_dec(x_15); +lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_4); +lean_dec(x_5); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_40 = !lean_is_exclusive(x_11); -if (x_40 == 0) +x_20 = !lean_is_exclusive(x_17); +if (x_20 == 0) { -lean_object* x_41; lean_object* x_42; -x_41 = lean_ctor_get(x_11, 0); -lean_dec(x_41); -x_42 = lean_box(0); -lean_ctor_set(x_11, 0, x_42); -return x_11; +return x_17; } else { -lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_43 = lean_ctor_get(x_11, 1); -lean_inc(x_43); -lean_dec(x_11); -x_44 = lean_box(0); -x_45 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_45, 0, x_44); -lean_ctor_set(x_45, 1, x_43); -return x_45; +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_17, 0); +x_22 = lean_ctor_get(x_17, 1); +lean_inc(x_22); +lean_inc(x_21); +lean_dec(x_17); +x_23 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_23, 0, x_21); +lean_ctor_set(x_23, 1, x_22); +return x_23; } } } } -LEAN_EXPORT lean_object* l_Lean_ForEachExprWhere_visit___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_10 = l_Lean_ForEachExprWhere_initCache; -x_11 = lean_st_mk_ref(x_10, x_9); +lean_object* x_11; +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_11) == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; 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_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6(x_1, x_2, x_4, x_3, x_12, x_5, x_6, x_7, x_8, x_13); -if (lean_obj_tag(x_14) == 0) -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_14 = l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_shouldInferResultUniverse___spec__1(x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_13); x_15 = lean_ctor_get(x_14, 0); lean_inc(x_15); x_16 = lean_ctor_get(x_14, 1); lean_inc(x_16); lean_dec(x_14); -x_17 = lean_st_ref_get(x_12, x_16); -lean_dec(x_12); -x_18 = !lean_is_exclusive(x_17); -if (x_18 == 0) +x_17 = l_Lean_Level_normalize(x_15); +lean_dec(x_15); +lean_inc(x_4); +lean_inc(x_17); +x_18 = l_Lean_Elab_Command_checkResultingUniverse(x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_16); +if (lean_obj_tag(x_18) == 0) { -lean_object* x_19; -x_19 = lean_ctor_get(x_17, 0); -lean_dec(x_19); -lean_ctor_set(x_17, 0, x_15); -return x_17; +uint8_t x_19; +x_19 = !lean_is_exclusive(x_18); +if (x_19 == 0) +{ +lean_object* x_20; lean_object* x_21; uint8_t x_22; +x_20 = lean_ctor_get(x_18, 1); +x_21 = lean_ctor_get(x_18, 0); +lean_dec(x_21); +x_22 = l_Lean_Level_isZero(x_17); +if (x_22 == 0) +{ +lean_object* x_23; +lean_free_object(x_18); +x_23 = l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses___spec__3(x_1, x_2, x_17, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_20); +return x_23; } else { -lean_object* x_20; lean_object* x_21; -x_20 = lean_ctor_get(x_17, 1); -lean_inc(x_20); +lean_object* x_24; lean_dec(x_17); -x_21 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_21, 0, x_15); -lean_ctor_set(x_21, 1, x_20); -return 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); +lean_dec(x_1); +x_24 = lean_box(0); +lean_ctor_set(x_18, 0, x_24); +return x_18; } } else { -uint8_t x_22; -lean_dec(x_12); -x_22 = !lean_is_exclusive(x_14); -if (x_22 == 0) +lean_object* x_25; uint8_t x_26; +x_25 = lean_ctor_get(x_18, 1); +lean_inc(x_25); +lean_dec(x_18); +x_26 = l_Lean_Level_isZero(x_17); +if (x_26 == 0) { -return x_14; +lean_object* x_27; +x_27 = l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses___spec__3(x_1, x_2, x_17, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_25); +return x_27; } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_14, 0); -x_24 = lean_ctor_get(x_14, 1); -lean_inc(x_24); -lean_inc(x_23); -lean_dec(x_14); -x_25 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_25, 0, x_23); -lean_ctor_set(x_25, 1, x_24); -return x_25; -} +lean_object* x_28; lean_object* x_29; +lean_dec(x_17); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +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_25); +return x_29; } } } -LEAN_EXPORT uint8_t l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__9___lambda__1(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; lean_object* x_4; uint8_t x_5; -x_3 = lean_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) +else { -uint8_t x_6; +uint8_t x_30; +lean_dec(x_17); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); -x_6 = 0; -return x_6; +lean_dec(x_2); +lean_dec(x_1); +x_30 = !lean_is_exclusive(x_18); +if (x_30 == 0) +{ +return x_18; } else { -size_t x_7; size_t x_8; uint8_t x_9; -x_7 = 0; -x_8 = lean_usize_of_nat(x_3); -lean_dec(x_3); -x_9 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__2(x_2, x_1, x_7, x_8); -return x_9; +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_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__9___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: +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; lean_object* x_22; uint8_t x_23; -x_12 = lean_unsigned_to_nat(0u); -x_13 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_6, x_12); -lean_inc(x_13); -x_14 = lean_mk_array(x_13, x_1); -x_15 = lean_unsigned_to_nat(1u); -x_16 = lean_nat_sub(x_13, x_15); -lean_dec(x_13); -x_17 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_6, x_14, x_16); -x_18 = lean_array_get_size(x_17); -x_19 = lean_box(0); -lean_inc(x_18); -x_20 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__3(x_2, x_3, x_17, x_18, x_18, x_4, x_18, x_15, x_19, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_17); -x_21 = lean_ctor_get(x_20, 1); -lean_inc(x_21); -lean_dec(x_20); -lean_inc(x_5); -x_22 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__4(x_2, x_5, x_18, x_5, x_15, x_19, x_7, x_8, x_9, x_10, x_21); +uint8_t x_34; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); lean_dec(x_5); -x_23 = !lean_is_exclusive(x_22); -if (x_23 == 0) +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_34 = !lean_is_exclusive(x_11); +if (x_34 == 0) { -lean_object* x_24; -x_24 = lean_ctor_get(x_22, 0); -lean_dec(x_24); -lean_ctor_set(x_22, 0, x_19); -return x_22; +return x_11; } else { -lean_object* x_25; lean_object* x_26; -x_25 = lean_ctor_get(x_22, 1); -lean_inc(x_25); -lean_dec(x_22); -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_19); -lean_ctor_set(x_26, 1, x_25); -return x_26; +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_11, 0); +x_36 = lean_ctor_get(x_11, 1); +lean_inc(x_36); +lean_inc(x_35); +lean_dec(x_11); +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_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, size_t x_8, size_t x_9, lean_object* x_10, 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_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses___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: { -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); +size_t x_15; size_t x_16; lean_object* x_17; +x_15 = lean_unbox_usize(x_5); lean_dec(x_5); +x_16 = lean_unbox_usize(x_6); +lean_dec(x_6); +x_17 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses___spec__1(x_1, x_2, x_3, x_4, x_15, x_16, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); lean_dec(x_1); -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_10); -lean_ctor_set(x_17, 1, x_15); return x_17; } +} +LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses___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_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses___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_6); +lean_dec(x_2); +return x_14; +} +} +LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUsed___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: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_8; lean_object* x_9; +x_8 = lean_box(0); +x_9 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_9, 0, x_8); +lean_ctor_set(x_9, 1, x_7); +return x_9; +} else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; +lean_object* 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); +x_11 = lean_ctor_get(x_1, 1); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_10, 1); +lean_inc(x_12); lean_dec(x_10); -x_18 = lean_ctor_get(x_7, 0); -x_19 = lean_array_uget(x_18, x_9); +x_13 = l_Lean_Expr_collectFVars(x_12, x_2, x_3, x_4, x_5, x_6, x_7); +x_14 = lean_ctor_get(x_13, 1); lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -x_20 = lean_infer_type(x_19, x_11, x_12, x_13, x_14, x_15); -if (lean_obj_tag(x_20) == 0) -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; lean_object* x_26; -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_20, 1); -lean_inc(x_22); -lean_dec(x_20); -lean_inc(x_2); -x_23 = lean_alloc_closure((void*)(l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__9___lambda__1___boxed), 2, 1); -lean_closure_set(x_23, 0, x_2); -lean_inc(x_3); -lean_inc(x_1); -lean_inc(x_6); -lean_inc(x_4); -lean_inc(x_5); -x_24 = lean_alloc_closure((void*)(l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__9___lambda__2___boxed), 11, 5); -lean_closure_set(x_24, 0, x_5); -lean_closure_set(x_24, 1, x_4); -lean_closure_set(x_24, 2, x_6); -lean_closure_set(x_24, 3, x_1); -lean_closure_set(x_24, 4, x_3); -x_25 = 1; -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -x_26 = l_Lean_ForEachExprWhere_visit___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__5(x_23, x_24, x_21, x_25, x_11, x_12, x_13, x_14, x_22); -if (lean_obj_tag(x_26) == 0) -{ -lean_object* x_27; size_t x_28; size_t x_29; lean_object* x_30; -x_27 = lean_ctor_get(x_26, 1); -lean_inc(x_27); -lean_dec(x_26); -x_28 = 1; -x_29 = lean_usize_add(x_9, x_28); -x_30 = lean_box(0); -x_9 = x_29; -x_10 = x_30; -x_15 = x_27; +lean_dec(x_13); +x_1 = x_11; +x_7 = x_14; goto _start; } +} +} +LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUsed___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: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_8; lean_object* x_9; +x_8 = lean_box(0); +x_9 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_9, 0, x_8); +lean_ctor_set(x_9, 1, x_7); +return x_9; +} else { -uint8_t x_32; -lean_dec(x_14); +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_10 = lean_ctor_get(x_1, 0); +lean_inc(x_10); +x_11 = lean_ctor_get(x_1, 1); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_10, 1); +lean_inc(x_12); +x_13 = l_Lean_Expr_collectFVars(x_12, x_2, x_3, x_4, x_5, x_6, x_7); +x_14 = lean_ctor_get(x_13, 1); +lean_inc(x_14); lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); +x_15 = lean_ctor_get(x_10, 2); +lean_inc(x_15); +lean_dec(x_10); +x_16 = l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUsed___spec__1(x_15, x_2, x_3, x_4, x_5, x_6, x_14); +x_17 = lean_ctor_get(x_16, 1); +lean_inc(x_17); +lean_dec(x_16); +x_1 = x_11; +x_7 = x_17; +goto _start; +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUsed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; +x_8 = l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUsed___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +return x_8; +} +} +LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUsed___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; +x_8 = l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUsed___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_32 = !lean_is_exclusive(x_26); -if (x_32 == 0) -{ -return x_26; +return x_8; } -else -{ -lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_33 = lean_ctor_get(x_26, 0); -x_34 = lean_ctor_get(x_26, 1); -lean_inc(x_34); -lean_inc(x_33); -lean_dec(x_26); -x_35 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_35, 0, x_33); -lean_ctor_set(x_35, 1, x_34); -return x_35; } +LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUsed___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; +x_8 = l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUsed___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_8; } } -else +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUsed___boxed(lean_object* x_1, 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_36; -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); +lean_object* x_8; +x_8 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUsed(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_36 = !lean_is_exclusive(x_20); -if (x_36 == 0) -{ -return x_20; +return x_8; } -else +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_removeUnused___closed__1() { +_start: { -lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_37 = lean_ctor_get(x_20, 0); -x_38 = lean_ctor_get(x_20, 1); -lean_inc(x_38); -lean_inc(x_37); -lean_dec(x_20); -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_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = lean_box(0); +x_2 = l_Lean_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__2___closed__3; +x_3 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__8___closed__1; +x_4 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_4, 0, x_2); +lean_ctor_set(x_4, 1, x_1); +lean_ctor_set(x_4, 2, x_3); +return x_4; } } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_removeUnused(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_10 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_removeUnused___closed__1; +x_11 = lean_st_mk_ref(x_10, 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 = l_List_forM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUsed___spec__2(x_2, x_12, x_5, x_6, x_7, x_8, 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_12, x_15); +lean_dec(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_Lean_Meta_removeUnused(x_1, x_17, x_5, x_6, x_7, x_8, x_18); +return x_19; } } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_removeUnused___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_removeUnused(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +return x_10; +} } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_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_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withUsed___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_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; 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___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_object* x_11; +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_removeUnused(x_1, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_11) == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_12, 1); lean_inc(x_13); -x_15 = lean_mk_array(x_13, x_14); -x_16 = lean_unsigned_to_nat(1u); -x_17 = lean_nat_sub(x_13, x_16); +x_14 = lean_ctor_get(x_11, 1); +lean_inc(x_14); +lean_dec(x_11); +x_15 = lean_ctor_get(x_12, 0); +lean_inc(x_15); +lean_dec(x_12); +x_16 = lean_ctor_get(x_13, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_13, 1); +lean_inc(x_17); lean_dec(x_13); -x_18 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_6, x_15, x_17); -x_19 = lean_box(0); -lean_inc(x_3); -lean_inc(x_2); -x_20 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__1(x_1, x_5, x_18, x_2, x_3, x_2, x_16, x_19, x_7, x_8, x_9, x_10, x_11); -x_21 = lean_ctor_get(x_20, 1); -lean_inc(x_21); -lean_dec(x_20); -x_22 = lean_array_get_size(x_5); -lean_inc(x_3); -x_23 = l_Array_toSubarray___rarg(x_5, x_3, x_22); -x_24 = lean_ctor_get(x_23, 2); -lean_inc(x_24); -x_25 = lean_usize_of_nat(x_24); -lean_dec(x_24); -x_26 = lean_ctor_get(x_23, 1); -lean_inc(x_26); -x_27 = lean_usize_of_nat(x_26); -lean_dec(x_26); -x_28 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__9(x_3, x_4, x_2, x_1, x_14, x_18, x_23, x_25, x_27, x_19, x_7, x_8, x_9, x_10, x_21); -lean_dec(x_23); -if (lean_obj_tag(x_28) == 0) +x_18 = lean_apply_1(x_3, x_17); +x_19 = l_Lean_Meta_withLCtx___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__3___rarg(x_15, x_16, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_14); +return x_19; +} +else { -uint8_t x_29; -x_29 = !lean_is_exclusive(x_28); -if (x_29 == 0) +uint8_t x_20; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_20 = !lean_is_exclusive(x_11); +if (x_20 == 0) { -lean_object* x_30; -x_30 = lean_ctor_get(x_28, 0); -lean_dec(x_30); -lean_ctor_set(x_28, 0, x_19); -return x_28; +return x_11; } else { -lean_object* x_31; lean_object* x_32; -x_31 = lean_ctor_get(x_28, 1); -lean_inc(x_31); -lean_dec(x_28); -x_32 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_32, 0, x_19); -lean_ctor_set(x_32, 1, x_31); -return x_32; +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; } } -else -{ -uint8_t x_33; -x_33 = !lean_is_exclusive(x_28); -if (x_33 == 0) -{ -return x_28; } -else +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withUsed(lean_object* x_1) { +_start: { -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_object* x_2; +x_2 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withUsed___rarg___boxed), 10, 0); +return x_2; } } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withUsed___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withUsed___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_1); +return x_11; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateParams___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: { -if (lean_obj_tag(x_5) == 0) +if (lean_obj_tag(x_2) == 0) { -lean_object* x_11; uint8_t x_12; +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_3); -lean_dec(x_2); -lean_dec(x_1); -x_11 = lean_st_ref_get(x_4, x_10); +lean_dec(x_5); lean_dec(x_4); -x_12 = !lean_is_exclusive(x_11); -if (x_12 == 0) -{ -return x_11; +lean_dec(x_1); +x_11 = l_List_reverse___rarg(x_3); +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; } 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_13; +x_13 = !lean_is_exclusive(x_2); +if (x_13 == 0) { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; lean_object* x_21; -x_16 = lean_ctor_get(x_5, 0); -lean_inc(x_16); -x_17 = lean_ctor_get(x_5, 1); -lean_inc(x_17); -lean_dec(x_5); -x_18 = lean_ctor_get(x_16, 1); -lean_inc(x_18); -lean_dec(x_16); -lean_inc(x_2); +lean_object* x_14; uint8_t x_15; +x_14 = lean_ctor_get(x_2, 0); +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; +x_16 = lean_ctor_get(x_2, 1); +x_17 = lean_ctor_get(x_14, 0); +x_18 = lean_ctor_get(x_14, 1); lean_inc(x_1); -lean_inc(x_3); -lean_inc(x_4); -x_19 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___lambda__1), 11, 4); -lean_closure_set(x_19, 0, x_4); -lean_closure_set(x_19, 1, x_3); -lean_closure_set(x_19, 2, x_1); -lean_closure_set(x_19, 3, x_2); -x_20 = 0; +x_19 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkTypeFor___lambda__1___boxed), 9, 2); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, x_18); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -x_21 = l_Lean_Meta_forallTelescopeReducing___at_Lean_Meta_getParamNames___spec__2___rarg(x_18, x_19, x_20, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_21) == 0) +lean_inc(x_5); +lean_inc(x_4); +x_20 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___rarg(x_1, x_19, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_20) == 0) { -lean_object* x_22; -x_22 = lean_ctor_get(x_21, 1); +lean_object* x_21; lean_object* x_22; +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_20, 1); lean_inc(x_22); -lean_dec(x_21); -x_5 = x_17; -x_10 = x_22; +lean_dec(x_20); +lean_ctor_set(x_14, 1, x_21); +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_22; +x_2 = _tmp_1; +x_3 = _tmp_2; +x_10 = _tmp_9; +} goto _start; } else { uint8_t x_24; +lean_free_object(x_14); lean_dec(x_17); +lean_free_object(x_2); +lean_dec(x_16); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); lean_dec(x_1); -x_24 = !lean_is_exclusive(x_21); +x_24 = !lean_is_exclusive(x_20); if (x_24 == 0) { -return x_21; +return x_20; } else { lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_21, 0); -x_26 = lean_ctor_get(x_21, 1); +x_25 = lean_ctor_get(x_20, 0); +x_26 = lean_ctor_get(x_20, 1); lean_inc(x_26); lean_inc(x_25); -lean_dec(x_21); +lean_dec(x_20); x_27 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_27, 0, x_25); lean_ctor_set(x_27, 1, x_26); @@ -24376,1529 +24962,1166 @@ return x_27; } } } +else +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_28 = lean_ctor_get(x_2, 1); +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); +lean_inc(x_1); +x_31 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkTypeFor___lambda__1___boxed), 9, 2); +lean_closure_set(x_31, 0, x_1); +lean_closure_set(x_31, 1, x_30); +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_32 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___rarg(x_1, x_31, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +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 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_35, 0, x_29); +lean_ctor_set(x_35, 1, x_33); +lean_ctor_set(x_2, 1, x_3); +lean_ctor_set(x_2, 0, x_35); +{ +lean_object* _tmp_1 = x_28; +lean_object* _tmp_2 = x_2; +lean_object* _tmp_9 = x_34; +x_2 = _tmp_1; +x_3 = _tmp_2; +x_10 = _tmp_9; } +goto _start; } -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { -_start: +else { -lean_object* x_14; -x_14 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); +lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; +lean_dec(x_29); +lean_free_object(x_2); +lean_dec(x_28); lean_dec(x_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_14; +x_37 = lean_ctor_get(x_32, 0); +lean_inc(x_37); +x_38 = lean_ctor_get(x_32, 1); +lean_inc(x_38); +if (lean_is_exclusive(x_32)) { + lean_ctor_release(x_32, 0); + lean_ctor_release(x_32, 1); + x_39 = x_32; +} else { + lean_dec_ref(x_32); + x_39 = lean_box(0); } +if (lean_is_scalar(x_39)) { + x_40 = lean_alloc_ctor(1, 2, 0); +} else { + x_40 = x_39; } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: +lean_ctor_set(x_40, 0, x_37); +lean_ctor_set(x_40, 1, x_38); +return x_40; +} +} +} +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_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__2(x_1, x_2, x_5, x_6); +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_2, 0); +x_42 = lean_ctor_get(x_2, 1); +lean_inc(x_42); +lean_inc(x_41); lean_dec(x_2); -lean_dec(x_1); -x_8 = lean_box(x_7); -return x_8; -} +x_43 = lean_ctor_get(x_41, 0); +lean_inc(x_43); +x_44 = lean_ctor_get(x_41, 1); +lean_inc(x_44); +if (lean_is_exclusive(x_41)) { + lean_ctor_release(x_41, 0); + lean_ctor_release(x_41, 1); + x_45 = x_41; +} else { + lean_dec_ref(x_41); + x_45 = lean_box(0); } -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___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) { -_start: +lean_inc(x_1); +x_46 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkTypeFor___lambda__1___boxed), 9, 2); +lean_closure_set(x_46, 0, x_1); +lean_closure_set(x_46, 1, x_44); +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_47 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___rarg(x_1, x_46, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_47) == 0) { -lean_object* x_15; -x_15 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___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); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_15; +lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_48 = lean_ctor_get(x_47, 0); +lean_inc(x_48); +x_49 = lean_ctor_get(x_47, 1); +lean_inc(x_49); +lean_dec(x_47); +if (lean_is_scalar(x_45)) { + x_50 = lean_alloc_ctor(0, 2, 0); +} else { + x_50 = x_45; } +lean_ctor_set(x_50, 0, x_43); +lean_ctor_set(x_50, 1, x_48); +x_51 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_51, 0, x_50); +lean_ctor_set(x_51, 1, x_3); +x_2 = x_42; +x_3 = x_51; +x_10 = x_49; +goto _start; } -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___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) { -_start: +else { -lean_object* x_12; -x_12 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_10); +lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; +lean_dec(x_45); +lean_dec(x_43); +lean_dec(x_42); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_1); -return x_12; -} -} -LEAN_EXPORT lean_object* l_Lean_ForEachExprWhere_visited___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; -x_8 = l_Lean_ForEachExprWhere_visited___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__7(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_8; -} -} -LEAN_EXPORT lean_object* l_Lean_ForEachExprWhere_checked___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; -x_8 = l_Lean_ForEachExprWhere_checked___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); -return x_8; -} +lean_dec(x_1); +x_53 = lean_ctor_get(x_47, 0); +lean_inc(x_53); +x_54 = lean_ctor_get(x_47, 1); +lean_inc(x_54); +if (lean_is_exclusive(x_47)) { + lean_ctor_release(x_47, 0); + lean_ctor_release(x_47, 1); + x_55 = x_47; +} else { + lean_dec_ref(x_47); + x_55 = lean_box(0); } -LEAN_EXPORT lean_object* l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___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_4); -lean_dec(x_4); -x_13 = l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6___lambda__1(x_1, x_2, x_3, x_12, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_6); -lean_dec(x_5); -return x_13; +if (lean_is_scalar(x_55)) { + x_56 = lean_alloc_ctor(1, 2, 0); +} else { + x_56 = x_55; } +lean_ctor_set(x_56, 0, x_53); +lean_ctor_set(x_56, 1, x_54); +return x_56; } -LEAN_EXPORT lean_object* l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_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: -{ -uint8_t x_11; lean_object* x_12; -x_11 = lean_unbox(x_3); -lean_dec(x_3); -x_12 = l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6(x_1, x_2, x_11, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_5); -return x_12; } } -LEAN_EXPORT lean_object* l_Lean_ForEachExprWhere_visit___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___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_4); -lean_dec(x_4); -x_11 = l_Lean_ForEachExprWhere_visit___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__5(x_1, x_2, x_3, x_10, x_5, x_6, x_7, x_8, x_9); -return x_11; } } -LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__9___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateParams___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: { -uint8_t x_3; lean_object* x_4; -x_3 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__9___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_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__9___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: +if (lean_obj_tag(x_2) == 0) { -lean_object* x_12; -x_12 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__9___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_10); +lean_object* x_11; lean_object* x_12; lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_1); +x_11 = l_List_reverse___rarg(x_3); +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_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { -_start: +else { -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_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__9(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); -return x_18; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask(lean_object* x_1, lean_object* x_2, lean_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_2); +if (x_13 == 0) { -lean_object* x_9; +lean_object* x_14; uint8_t x_15; +x_14 = lean_ctor_get(x_2, 0); +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; uint8_t x_20; uint8_t x_21; uint8_t x_22; lean_object* x_23; +x_16 = lean_ctor_get(x_2, 1); +x_17 = lean_ctor_get(x_14, 0); +x_18 = lean_ctor_get(x_14, 1); +x_19 = lean_ctor_get(x_14, 2); +x_20 = 0; +x_21 = 1; +x_22 = 1; +lean_inc(x_1); +x_23 = l_Lean_Meta_mkForallFVars(x_1, x_18, x_20, x_21, x_22, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_23) == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +x_26 = lean_box(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); -lean_inc(x_2); -x_9 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getArity(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_inc(x_1); +x_27 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateParams___spec__1(x_1, x_19, x_26, x_4, x_5, x_6, x_7, x_8, x_9, x_25); +if (lean_obj_tag(x_27) == 0) { -lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_11 = lean_ctor_get(x_9, 0); -x_12 = lean_ctor_get(x_9, 1); -x_13 = lean_nat_dec_le(x_11, x_1); -if (x_13 == 0) +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); +lean_ctor_set(x_14, 2, x_28); +lean_ctor_set(x_14, 1, x_24); +lean_ctor_set(x_2, 1, x_3); { -uint8_t x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -lean_free_object(x_9); -x_14 = 0; -x_15 = lean_box(x_14); -lean_inc(x_1); -x_16 = lean_mk_array(x_1, x_15); -x_17 = lean_nat_sub(x_11, x_1); -x_18 = 1; -x_19 = lean_box(x_18); -x_20 = lean_mk_array(x_17, x_19); -x_21 = l_Array_append___rarg(x_16, x_20); -lean_dec(x_20); -x_22 = lean_st_mk_ref(x_21, x_12); -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_2, 2); -lean_inc(x_25); -lean_dec(x_2); -x_26 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go(x_1, x_3, x_11, x_23, x_25, x_4, x_5, x_6, x_7, x_24); -return x_26; +lean_object* _tmp_1 = x_16; +lean_object* _tmp_2 = x_2; +lean_object* _tmp_9 = x_29; +x_2 = _tmp_1; +x_3 = _tmp_2; +x_10 = _tmp_9; +} +goto _start; } else { -uint8_t x_27; lean_object* x_28; lean_object* x_29; +uint8_t x_31; +lean_dec(x_24); +lean_free_object(x_14); +lean_dec(x_17); +lean_free_object(x_2); +lean_dec(x_16); +lean_dec(x_9); +lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); lean_dec(x_1); -x_27 = 0; -x_28 = lean_box(x_27); -x_29 = lean_mk_array(x_11, x_28); -lean_ctor_set(x_9, 0, x_29); -return x_9; -} -} -else -{ -lean_object* x_30; lean_object* x_31; uint8_t x_32; -x_30 = lean_ctor_get(x_9, 0); -x_31 = lean_ctor_get(x_9, 1); -lean_inc(x_31); -lean_inc(x_30); -lean_dec(x_9); -x_32 = lean_nat_dec_le(x_30, x_1); -if (x_32 == 0) +x_31 = !lean_is_exclusive(x_27); +if (x_31 == 0) { -uint8_t x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_33 = 0; -x_34 = lean_box(x_33); -lean_inc(x_1); -x_35 = lean_mk_array(x_1, x_34); -x_36 = lean_nat_sub(x_30, x_1); -x_37 = 1; -x_38 = lean_box(x_37); -x_39 = lean_mk_array(x_36, x_38); -x_40 = l_Array_append___rarg(x_35, x_39); -lean_dec(x_39); -x_41 = lean_st_mk_ref(x_40, x_31); -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_2, 2); -lean_inc(x_44); -lean_dec(x_2); -x_45 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go(x_1, x_3, x_30, x_42, x_44, x_4, x_5, x_6, x_7, x_43); -return x_45; +return x_27; } else { -uint8_t x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_46 = 0; -x_47 = lean_box(x_46); -x_48 = lean_mk_array(x_30, x_47); -x_49 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_49, 0, x_48); -lean_ctor_set(x_49, 1, x_31); -return x_49; +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; } } } else { -uint8_t x_50; +uint8_t x_35; +lean_free_object(x_14); +lean_dec(x_19); +lean_dec(x_17); +lean_free_object(x_2); +lean_dec(x_16); +lean_dec(x_9); +lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); lean_dec(x_1); -x_50 = !lean_is_exclusive(x_9); -if (x_50 == 0) +x_35 = !lean_is_exclusive(x_23); +if (x_35 == 0) { -return x_9; +return x_23; } else { -lean_object* x_51; lean_object* x_52; lean_object* x_53; -x_51 = lean_ctor_get(x_9, 0); -x_52 = lean_ctor_get(x_9, 1); -lean_inc(x_52); -lean_inc(x_51); -lean_dec(x_9); -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_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_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isDomainDefEq(lean_object* x_1, 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; -x_8 = l_Lean_Expr_isForall(x_1); -if (x_8 == 0) +lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; uint8_t x_44; uint8_t x_45; lean_object* x_46; +x_39 = lean_ctor_get(x_2, 1); +x_40 = lean_ctor_get(x_14, 0); +x_41 = lean_ctor_get(x_14, 1); +x_42 = lean_ctor_get(x_14, 2); +lean_inc(x_42); +lean_inc(x_41); +lean_inc(x_40); +lean_dec(x_14); +x_43 = 0; +x_44 = 1; +x_45 = 1; +lean_inc(x_1); +x_46 = l_Lean_Meta_mkForallFVars(x_1, x_41, x_43, x_44, x_45, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_46) == 0) { -uint8_t x_9; lean_object* x_10; lean_object* x_11; -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_9 = 0; -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; -} -else +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +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_box(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); +lean_inc(x_1); +x_50 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateParams___spec__1(x_1, x_42, x_49, x_4, x_5, x_6, x_7, x_8, x_9, x_48); +if (lean_obj_tag(x_50) == 0) { -lean_object* x_12; lean_object* x_13; -x_12 = l_Lean_Expr_bindingDomain_x21(x_1); -x_13 = l_Lean_Meta_isExprDefEq(x_12, x_2, x_3, x_4, x_5, x_6, x_7); -return x_13; -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isDomainDefEq___boxed(lean_object* x_1, 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_51; lean_object* x_52; lean_object* x_53; +x_51 = lean_ctor_get(x_50, 0); +lean_inc(x_51); +x_52 = lean_ctor_get(x_50, 1); +lean_inc(x_52); +lean_dec(x_50); +x_53 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_53, 0, x_40); +lean_ctor_set(x_53, 1, x_47); +lean_ctor_set(x_53, 2, x_51); +lean_ctor_set(x_2, 1, x_3); +lean_ctor_set(x_2, 0, x_53); { -lean_object* x_8; -x_8 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isDomainDefEq(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -lean_dec(x_1); -return x_8; +lean_object* _tmp_1 = x_39; +lean_object* _tmp_2 = x_2; +lean_object* _tmp_9 = x_52; +x_2 = _tmp_1; +x_3 = _tmp_2; +x_10 = _tmp_9; } +goto _start; } -LEAN_EXPORT lean_object* l_List_allM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_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: -{ -if (lean_obj_tag(x_2) == 0) +else { -uint8_t x_8; lean_object* x_9; lean_object* x_10; +lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; +lean_dec(x_47); +lean_dec(x_40); +lean_free_object(x_2); +lean_dec(x_39); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_8 = 1; -x_9 = lean_box(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_7); -return x_10; -} -else -{ -lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_11 = lean_ctor_get(x_2, 0); -x_12 = lean_ctor_get(x_2, 1); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_1); -x_13 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isDomainDefEq(x_11, x_1, x_3, x_4, x_5, x_6, x_7); -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; -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_16 = !lean_is_exclusive(x_13); -if (x_16 == 0) -{ -lean_object* x_17; uint8_t x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_13, 0); -lean_dec(x_17); -x_18 = 0; -x_19 = lean_box(x_18); -lean_ctor_set(x_13, 0, x_19); -return x_13; -} -else -{ -lean_object* x_20; uint8_t x_21; lean_object* x_22; lean_object* x_23; -x_20 = lean_ctor_get(x_13, 1); -lean_inc(x_20); -lean_dec(x_13); -x_21 = 0; -x_22 = lean_box(x_21); -x_23 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_23, 0, x_22); -lean_ctor_set(x_23, 1, x_20); -return x_23; +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; } -else -{ -lean_object* x_24; -x_24 = lean_ctor_get(x_13, 1); -lean_inc(x_24); -lean_dec(x_13); -x_2 = x_12; -x_7 = x_24; -goto _start; +lean_ctor_set(x_58, 0, x_55); +lean_ctor_set(x_58, 1, x_56); +return x_58; } } else { -uint8_t x_26; +lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; +lean_dec(x_42); +lean_dec(x_40); +lean_free_object(x_2); +lean_dec(x_39); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); 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; -} +x_59 = lean_ctor_get(x_46, 0); +lean_inc(x_59); +x_60 = lean_ctor_get(x_46, 1); +lean_inc(x_60); +if (lean_is_exclusive(x_46)) { + lean_ctor_release(x_46, 0); + lean_ctor_release(x_46, 1); + x_61 = x_46; +} else { + lean_dec_ref(x_46); + x_61 = lean_box(0); } +if (lean_is_scalar(x_61)) { + x_62 = lean_alloc_ctor(1, 2, 0); +} else { + x_62 = x_61; } +lean_ctor_set(x_62, 0, x_59); +lean_ctor_set(x_62, 1, x_60); +return x_62; } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -if (lean_obj_tag(x_2) == 0) -{ -lean_object* x_9; lean_object* x_10; -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -x_9 = l_List_reverse___rarg(x_3); -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_9); -lean_ctor_set(x_10, 1, x_8); -return x_10; } else { -uint8_t x_11; -x_11 = !lean_is_exclusive(x_2); -if (x_11 == 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; uint8_t x_69; uint8_t x_70; uint8_t x_71; lean_object* x_72; +x_63 = lean_ctor_get(x_2, 0); +x_64 = lean_ctor_get(x_2, 1); +lean_inc(x_64); +lean_inc(x_63); +lean_dec(x_2); +x_65 = lean_ctor_get(x_63, 0); +lean_inc(x_65); +x_66 = lean_ctor_get(x_63, 1); +lean_inc(x_66); +x_67 = lean_ctor_get(x_63, 2); +lean_inc(x_67); +if (lean_is_exclusive(x_63)) { + lean_ctor_release(x_63, 0); + lean_ctor_release(x_63, 1); + lean_ctor_release(x_63, 2); + x_68 = x_63; +} else { + lean_dec_ref(x_63); + x_68 = lean_box(0); +} +x_69 = 0; +x_70 = 1; +x_71 = 1; +lean_inc(x_1); +x_72 = l_Lean_Meta_mkForallFVars(x_1, x_66, x_69, x_70, x_71, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_72) == 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); -x_13 = lean_ctor_get(x_2, 1); -x_14 = l_Lean_Expr_bindingBody_x21(x_12); -lean_dec(x_12); -x_15 = lean_expr_instantiate1(x_14, x_1); -lean_dec(x_14); +lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; +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_box(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_16 = l_Lean_Meta_whnfD(x_15, 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; -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_2, 1, x_3); -lean_ctor_set(x_2, 0, x_17); +lean_inc(x_1); +x_76 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateParams___spec__1(x_1, x_67, x_75, x_4, x_5, x_6, x_7, x_8, x_9, x_74); +if (lean_obj_tag(x_76) == 0) { -lean_object* _tmp_1 = x_13; -lean_object* _tmp_2 = x_2; -lean_object* _tmp_7 = x_18; -x_2 = _tmp_1; -x_3 = _tmp_2; -x_8 = _tmp_7; +lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; +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); +if (lean_is_scalar(x_68)) { + x_79 = lean_alloc_ctor(0, 3, 0); +} else { + x_79 = x_68; } +lean_ctor_set(x_79, 0, x_65); +lean_ctor_set(x_79, 1, x_73); +lean_ctor_set(x_79, 2, x_77); +x_80 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_80, 0, x_79); +lean_ctor_set(x_80, 1, x_3); +x_2 = x_64; +x_3 = x_80; +x_10 = x_78; goto _start; } else { -uint8_t x_20; -lean_free_object(x_2); -lean_dec(x_13); +lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; +lean_dec(x_73); +lean_dec(x_68); +lean_dec(x_65); +lean_dec(x_64); +lean_dec(x_9); +lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_20 = !lean_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; +lean_dec(x_1); +x_82 = lean_ctor_get(x_76, 0); +lean_inc(x_82); +x_83 = lean_ctor_get(x_76, 1); +lean_inc(x_83); +if (lean_is_exclusive(x_76)) { + lean_ctor_release(x_76, 0); + lean_ctor_release(x_76, 1); + 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(1, 2, 0); +} else { + x_85 = x_84; } +lean_ctor_set(x_85, 0, x_82); +lean_ctor_set(x_85, 1, x_83); +return x_85; } -else -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_24 = lean_ctor_get(x_2, 0); -x_25 = lean_ctor_get(x_2, 1); -lean_inc(x_25); -lean_inc(x_24); -lean_dec(x_2); -x_26 = l_Lean_Expr_bindingBody_x21(x_24); -lean_dec(x_24); -x_27 = lean_expr_instantiate1(x_26, x_1); -lean_dec(x_26); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -x_28 = l_Lean_Meta_whnfD(x_27, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_28) == 0) -{ -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_28, 0); -lean_inc(x_29); -x_30 = lean_ctor_get(x_28, 1); -lean_inc(x_30); -lean_dec(x_28); -x_31 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_31, 0, x_29); -lean_ctor_set(x_31, 1, x_3); -x_2 = x_25; -x_3 = x_31; -x_8 = x_30; -goto _start; } else { -lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; -lean_dec(x_25); +lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; +lean_dec(x_68); +lean_dec(x_67); +lean_dec(x_65); +lean_dec(x_64); +lean_dec(x_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_33 = lean_ctor_get(x_28, 0); -lean_inc(x_33); -x_34 = lean_ctor_get(x_28, 1); -lean_inc(x_34); -if (lean_is_exclusive(x_28)) { - lean_ctor_release(x_28, 0); - lean_ctor_release(x_28, 1); - x_35 = x_28; +lean_dec(x_1); +x_86 = lean_ctor_get(x_72, 0); +lean_inc(x_86); +x_87 = lean_ctor_get(x_72, 1); +lean_inc(x_87); +if (lean_is_exclusive(x_72)) { + lean_ctor_release(x_72, 0); + lean_ctor_release(x_72, 1); + x_88 = x_72; } else { - lean_dec_ref(x_28); - x_35 = lean_box(0); + lean_dec_ref(x_72); + x_88 = lean_box(0); } -if (lean_is_scalar(x_35)) { - x_36 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_88)) { + x_89 = lean_alloc_ctor(1, 2, 0); } else { - x_36 = x_35; + x_89 = x_88; } -lean_ctor_set(x_36, 0, x_33); -lean_ctor_set(x_36, 1, x_34); -return x_36; +lean_ctor_set(x_89, 0, x_86); +lean_ctor_set(x_89, 1, x_87); +return x_89; } } } } } -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___spec__3(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateParams(lean_object* x_1, lean_object* x_2, lean_object* x_3, 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_5; -x_5 = lean_usize_dec_eq(x_3, x_4); -if (x_5 == 0) -{ -lean_object* x_6; lean_object* x_7; uint8_t x_8; -x_6 = lean_array_uget(x_2, x_3); -x_7 = lean_array_get_size(x_6); -x_8 = lean_nat_dec_lt(x_1, x_7); -lean_dec(x_7); -if (x_8 == 0) -{ -uint8_t x_9; -lean_dec(x_6); -x_9 = 1; -return x_9; +lean_object* x_10; lean_object* x_11; +x_10 = lean_box(0); +x_11 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateParams___spec__2(x_1, x_2, x_10, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_11; } -else +} +LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectLevelParamsInInductive___spec__1(lean_object* x_1, lean_object* x_2) { +_start: { -lean_object* x_10; uint8_t x_11; -x_10 = lean_array_fget(x_6, x_1); -lean_dec(x_6); -x_11 = lean_unbox(x_10); -lean_dec(x_10); -if (x_11 == 0) +if (lean_obj_tag(x_1) == 0) { -uint8_t x_12; -x_12 = 1; -return x_12; +return x_2; } else { -size_t x_13; size_t x_14; -x_13 = 1; -x_14 = lean_usize_add(x_3, x_13); -x_3 = x_14; +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); +x_4 = lean_ctor_get(x_1, 1); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_ctor_get(x_3, 1); +lean_inc(x_5); +lean_dec(x_3); +x_6 = l_Lean_CollectLevelParams_main(x_5, x_2); +x_1 = x_4; +x_2 = x_6; goto _start; } } } -else -{ -uint8_t x_16; -x_16 = 0; -return x_16; -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_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) { -_start: -{ -lean_object* x_8; -x_8 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_8, 0, x_1); -lean_ctor_set(x_8, 1, x_7); -return x_8; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_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_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectLevelParamsInInductive___spec__2(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_12; lean_object* x_13; -x_12 = lean_box(0); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -x_13 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___spec__2(x_6, x_1, x_12, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_13) == 0) -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_14 = lean_ctor_get(x_13, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_13, 1); -lean_inc(x_15); -lean_dec(x_13); -x_16 = lean_unsigned_to_nat(1u); -x_17 = lean_nat_add(x_2, x_16); -x_18 = l_Lean_Expr_bindingBody_x21(x_3); -x_19 = lean_expr_instantiate1(x_18, x_6); -lean_dec(x_18); -x_20 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go(x_4, x_5, x_17, x_19, x_14, x_7, x_8, x_9, x_10, x_15); -return x_20; -} -else -{ -uint8_t x_21; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_5); -lean_dec(x_4); -x_21 = !lean_is_exclusive(x_13); -if (x_21 == 0) +if (lean_obj_tag(x_1) == 0) { -return x_13; +return x_2; } else { -lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_22 = lean_ctor_get(x_13, 0); -x_23 = lean_ctor_get(x_13, 1); -lean_inc(x_23); -lean_inc(x_22); -lean_dec(x_13); -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; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_3 = lean_ctor_get(x_1, 0); +lean_inc(x_3); +x_4 = lean_ctor_get(x_1, 1); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_ctor_get(x_3, 1); +lean_inc(x_5); +x_6 = l_Lean_CollectLevelParams_main(x_5, x_2); +x_7 = lean_ctor_get(x_3, 2); +lean_inc(x_7); +lean_dec(x_3); +x_8 = l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectLevelParamsInInductive___spec__1(x_7, x_6); +x_1 = x_4; +x_2 = x_8; +goto _start; } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__3___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("a", 1, 1); -return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__3___closed__2() { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectLevelParamsInInductive___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_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__3___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); +x_1 = l_Lean_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__2___closed__3; +x_2 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__8___closed__1; +x_3 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_1); +lean_ctor_set(x_3, 2, x_2); return x_3; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_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_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectLevelParamsInInductive(lean_object* x_1) { _start: { -lean_object* x_13; lean_object* x_14; uint8_t x_15; uint8_t x_16; lean_object* x_17; -x_13 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__2___boxed), 11, 5); -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); -x_14 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__3___closed__2; -x_15 = 0; -x_16 = 0; -x_17 = l_Lean_Meta_withLocalDecl___at_Lean_Meta_forallTelescopeCompatibleAux___spec__15___rarg(x_14, x_15, x_6, x_13, x_16, x_8, x_9, x_10, x_11, x_12); -return x_17; +lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_2 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectLevelParamsInInductive___closed__1; +x_3 = l_List_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectLevelParamsInInductive___spec__2(x_1, x_2); +x_4 = lean_ctor_get(x_3, 2); +lean_inc(x_4); +lean_dec(x_3); +return x_4; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4___closed__1() { +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkIndFVar2Const___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_1; -x_1 = lean_mk_string_unchecked("domain not def eq: ", 19, 19); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4___closed__2() { -_start: +uint8_t x_11; +x_11 = lean_nat_dec_le(x_8, x_7); +if (x_11 == 0) { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4___closed__3() { -_start: +lean_object* x_12; uint8_t x_13; +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_nat_dec_eq(x_6, x_12); +if (x_13 == 0) { -lean_object* x_1; -x_1 = lean_mk_string_unchecked(", ", 2, 2); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4___closed__4() { -_start: +lean_object* x_14; lean_object* x_15; uint8_t x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; +x_14 = lean_unsigned_to_nat(1u); +x_15 = lean_nat_sub(x_6, x_14); +lean_dec(x_6); +x_16 = lean_nat_dec_lt(x_7, x_5); +x_17 = lean_array_get_size(x_2); +x_18 = lean_nat_dec_lt(x_7, x_17); +lean_dec(x_17); +if (x_16 == 0) { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4___closed__3; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} +lean_object* x_71; lean_object* x_72; +x_71 = l_Lean_Elab_Command_instInhabitedInductiveView; +x_72 = l_outOfBounds___rarg(x_71); +x_19 = x_72; +goto block_70; } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4___closed__5() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked(" =\?= ", 5, 5); -return x_1; -} +lean_object* x_73; +x_73 = lean_array_fget(x_1, x_7); +x_19 = x_73; +goto block_70; } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4___closed__6() { -_start: +block_70: { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4___closed__5; -x_2 = l_Lean_stringToMessageData(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; +x_20 = lean_ctor_get(x_19, 4); +lean_inc(x_20); +lean_dec(x_19); +lean_inc(x_3); +x_21 = l_Lean_Expr_const___override(x_20, x_3); +if (x_18 == 0) +{ +lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; +x_63 = l_Lean_instInhabitedExpr; +x_64 = l_outOfBounds___rarg(x_63); +x_65 = lean_ctor_get(x_10, 0); +lean_inc(x_65); +x_66 = lean_ctor_get(x_10, 1); +lean_inc(x_66); +lean_dec(x_10); +x_22 = x_64; +x_23 = x_65; +x_24 = x_66; +goto block_62; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: +else { -lean_object* x_12; lean_object* x_13; -x_12 = l_Lean_Expr_bindingDomain_x21(x_1); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_12); -x_13 = l_List_allM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___spec__1(x_12, x_2, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_13) == 0) +lean_object* x_67; lean_object* x_68; lean_object* x_69; +x_67 = lean_array_fget(x_2, x_7); +x_68 = lean_ctor_get(x_10, 0); +lean_inc(x_68); +x_69 = lean_ctor_get(x_10, 1); +lean_inc(x_69); +lean_dec(x_10); +x_22 = x_67; +x_23 = x_68; +x_24 = x_69; +goto block_62; +} +block_62: { -lean_object* x_14; uint8_t x_15; -x_14 = lean_ctor_get(x_13, 0); -lean_inc(x_14); -x_15 = lean_unbox(x_14); -lean_dec(x_14); -if (x_15 == 0) +lean_object* x_25; uint64_t x_26; uint64_t x_27; uint64_t x_28; uint64_t x_29; uint64_t x_30; uint64_t x_31; uint64_t x_32; size_t x_33; size_t x_34; size_t x_35; size_t x_36; size_t x_37; lean_object* x_38; uint8_t x_39; +x_25 = lean_array_get_size(x_24); +x_26 = l_Lean_Expr_hash(x_22); +x_27 = 32; +x_28 = lean_uint64_shift_right(x_26, x_27); +x_29 = lean_uint64_xor(x_26, x_28); +x_30 = 16; +x_31 = lean_uint64_shift_right(x_29, x_30); +x_32 = lean_uint64_xor(x_29, x_31); +x_33 = lean_uint64_to_usize(x_32); +x_34 = lean_usize_of_nat(x_25); +lean_dec(x_25); +x_35 = 1; +x_36 = lean_usize_sub(x_34, x_35); +x_37 = lean_usize_land(x_33, x_36); +x_38 = lean_array_uget(x_24, x_37); +x_39 = l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Elab_DeclNameGen_0__Lean_Elab_Command_NameGen_winnowExpr_visit___spec__1(x_22, x_38); +if (x_39 == 0) { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); -x_16 = lean_ctor_get(x_13, 1); -lean_inc(x_16); -lean_dec(x_13); -x_17 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__3; -x_18 = l_Lean_isTracingEnabledFor___at_Lean_Meta_processPostponed_loop___spec__1(x_17, x_7, x_8, x_9, x_10, x_16); -x_19 = lean_ctor_get(x_18, 0); -lean_inc(x_19); -x_20 = lean_unbox(x_19); -lean_dec(x_19); -if (x_20 == 0) +lean_object* x_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; +x_40 = lean_nat_add(x_23, x_14); +lean_dec(x_23); +x_41 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_41, 0, x_22); +lean_ctor_set(x_41, 1, x_21); +lean_ctor_set(x_41, 2, x_38); +x_42 = lean_array_uset(x_24, x_37, x_41); +x_43 = lean_unsigned_to_nat(4u); +x_44 = lean_nat_mul(x_40, x_43); +x_45 = lean_unsigned_to_nat(3u); +x_46 = lean_nat_div(x_44, x_45); +lean_dec(x_44); +x_47 = lean_array_get_size(x_42); +x_48 = lean_nat_dec_le(x_46, x_47); +lean_dec(x_47); +lean_dec(x_46); +if (x_48 == 0) { -uint8_t x_21; -lean_dec(x_12); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); +lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_49 = l_Std_DHashMap_Internal_Raw_u2080_expand___at___private_Lean_Elab_DeclNameGen_0__Lean_Elab_Command_NameGen_winnowExpr_visit___spec__2(x_42); +x_50 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_50, 0, x_40); +lean_ctor_set(x_50, 1, x_49); +x_51 = lean_nat_add(x_7, x_9); lean_dec(x_7); -lean_dec(x_1); -x_21 = !lean_is_exclusive(x_18); -if (x_21 == 0) -{ -lean_object* x_22; -x_22 = lean_ctor_get(x_18, 0); -lean_dec(x_22); -lean_ctor_set(x_18, 0, x_3); -return x_18; +x_6 = x_15; +x_7 = x_51; +x_10 = x_50; +goto _start; } else { -lean_object* x_23; lean_object* x_24; -x_23 = lean_ctor_get(x_18, 1); -lean_inc(x_23); -lean_dec(x_18); -x_24 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_24, 0, x_3); -lean_ctor_set(x_24, 1, x_23); -return x_24; +lean_object* x_53; lean_object* x_54; +x_53 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_53, 0, x_40); +lean_ctor_set(x_53, 1, x_42); +x_54 = lean_nat_add(x_7, x_9); +lean_dec(x_7); +x_6 = x_15; +x_7 = x_54; +x_10 = x_53; +goto _start; } } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; -x_25 = lean_ctor_get(x_18, 1); -lean_inc(x_25); -lean_dec(x_18); -lean_inc(x_3); -x_26 = l___private_Init_Data_Repr_0__Nat_reprFast(x_3); -x_27 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_27, 0, x_26); -x_28 = l_Lean_MessageData_ofFormat(x_27); -x_29 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4___closed__2; -x_30 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_30, 0, x_29); -lean_ctor_set(x_30, 1, x_28); -x_31 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4___closed__4; -x_32 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_32, 0, x_30); -lean_ctor_set(x_32, 1, x_31); -x_33 = l_Lean_MessageData_ofExpr(x_1); -x_34 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_34, 0, x_32); -lean_ctor_set(x_34, 1, x_33); -x_35 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4___closed__6; -x_36 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_36, 0, x_34); -lean_ctor_set(x_36, 1, x_35); -x_37 = l_Lean_MessageData_ofExpr(x_12); -x_38 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -x_39 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5; -x_40 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_40, 0, x_38); -lean_ctor_set(x_40, 1, x_39); -x_41 = l_Lean_addTrace___at_Lean_Meta_processPostponed_loop___spec__2(x_17, x_40, x_7, x_8, x_9, x_10, x_25); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); +lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; +lean_inc(x_4); +x_56 = lean_array_uset(x_24, x_37, x_4); +x_57 = l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Elab_DeclNameGen_0__Lean_Elab_Command_NameGen_winnowExpr_visit___spec__5(x_22, x_21, x_38); +x_58 = lean_array_uset(x_56, x_37, x_57); +x_59 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_59, 0, x_23); +lean_ctor_set(x_59, 1, x_58); +x_60 = lean_nat_add(x_7, x_9); lean_dec(x_7); -x_42 = !lean_is_exclusive(x_41); -if (x_42 == 0) -{ -lean_object* x_43; -x_43 = lean_ctor_get(x_41, 0); -lean_dec(x_43); -lean_ctor_set(x_41, 0, x_3); -return x_41; +x_6 = x_15; +x_7 = x_60; +x_10 = x_59; +goto _start; } -else -{ -lean_object* x_44; lean_object* x_45; -x_44 = lean_ctor_get(x_41, 1); -lean_inc(x_44); -lean_dec(x_41); -x_45 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_45, 0, x_3); -lean_ctor_set(x_45, 1, x_44); -return x_45; } } } else { -lean_object* x_46; lean_object* x_47; lean_object* x_48; -x_46 = lean_ctor_get(x_13, 1); -lean_inc(x_46); -lean_dec(x_13); -x_47 = lean_box(0); -x_48 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__3(x_2, x_3, x_1, x_4, x_5, x_12, x_47, x_7, x_8, x_9, x_10, x_46); -return x_48; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_4); +lean_dec(x_3); +return x_10; } } else { -uint8_t x_49; -lean_dec(x_12); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); lean_dec(x_7); -lean_dec(x_5); +lean_dec(x_6); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_49 = !lean_is_exclusive(x_13); -if (x_49 == 0) -{ -return x_13; +return x_10; } -else -{ -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_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; } } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkIndFVar2Const(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 = lean_box(0); +x_5 = l_List_mapTR_loop___at_Lean_mkConstWithLevelParams___spec__1(x_3, x_4); +x_6 = lean_box(0); +x_7 = lean_array_get_size(x_1); +x_8 = lean_unsigned_to_nat(0u); +x_9 = lean_unsigned_to_nat(1u); +x_10 = l_Lean_localDeclDependsOnPred___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__2___closed__3; +lean_inc(x_7); +x_11 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkIndFVar2Const___spec__1(x_1, x_2, x_5, x_6, x_7, x_7, x_8, x_7, x_9, x_10); +lean_dec(x_7); +return x_11; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkIndFVar2Const___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -uint8_t x_12; -x_12 = l_Lean_Expr_isForall(x_1); -if (x_12 == 0) -{ -lean_object* x_13; -lean_dec(x_10); +lean_object* x_11; +x_11 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkIndFVar2Const___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_5); -lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_3); -lean_ctor_set(x_13, 1, x_11); -return x_13; +return x_11; } -else -{ -lean_object* x_14; lean_object* x_15; -x_14 = lean_box(0); -x_15 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4(x_1, x_2, x_3, x_4, x_5, x_14, x_7, x_8, x_9, x_10, x_11); -return x_15; } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkIndFVar2Const___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkIndFVar2Const(x_1, x_2, x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_4; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_11; uint8_t x_12; -x_11 = lean_array_get_size(x_2); -x_12 = lean_nat_dec_lt(x_3, x_11); -lean_dec(x_11); -if (x_12 == 0) +uint8_t x_5; +x_5 = l_Lean_Expr_isFVar(x_4); +if (x_5 == 0) { -lean_object* x_13; -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_3); -lean_ctor_set(x_13, 1, x_10); -return x_13; +lean_object* x_6; +x_6 = lean_box(0); +return x_6; } else { -lean_object* x_14; lean_object* x_15; uint8_t x_16; -x_14 = lean_array_get_size(x_1); -x_15 = lean_unsigned_to_nat(0u); -x_16 = lean_nat_dec_lt(x_15, x_14); -if (x_16 == 0) +lean_object* x_7; lean_object* x_8; uint64_t x_9; uint64_t x_10; uint64_t x_11; uint64_t x_12; uint64_t x_13; uint64_t x_14; uint64_t x_15; size_t x_16; size_t x_17; size_t x_18; size_t x_19; size_t x_20; lean_object* x_21; lean_object* x_22; +x_7 = lean_ctor_get(x_1, 1); +x_8 = lean_array_get_size(x_7); +x_9 = l_Lean_Expr_hash(x_4); +x_10 = 32; +x_11 = lean_uint64_shift_right(x_9, x_10); +x_12 = lean_uint64_xor(x_9, x_11); +x_13 = 16; +x_14 = lean_uint64_shift_right(x_12, x_13); +x_15 = lean_uint64_xor(x_12, x_14); +x_16 = lean_uint64_to_usize(x_15); +x_17 = lean_usize_of_nat(x_8); +lean_dec(x_8); +x_18 = 1; +x_19 = lean_usize_sub(x_17, x_18); +x_20 = lean_usize_land(x_16, x_19); +x_21 = lean_array_uget(x_7, x_20); +x_22 = l_Std_DHashMap_Internal_AssocList_get_x3f___at___private_Lean_Elab_DeclNameGen_0__Lean_Elab_Command_NameGen_winnowExpr_visit___spec__6(x_4, x_21); +lean_dec(x_21); +if (lean_obj_tag(x_22) == 0) { -lean_object* x_17; lean_object* x_18; -lean_dec(x_14); -x_17 = lean_box(0); -x_18 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__5(x_4, x_5, x_3, x_1, x_2, x_17, x_6, x_7, x_8, x_9, x_10); -return x_18; +lean_object* x_23; +x_23 = lean_box(0); +return x_23; } else { -size_t x_19; size_t x_20; uint8_t x_21; -x_19 = 0; -x_20 = lean_usize_of_nat(x_14); -lean_dec(x_14); -x_21 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___spec__3(x_3, x_1, x_19, x_20); -if (x_21 == 0) +uint8_t x_24; +x_24 = !lean_is_exclusive(x_22); +if (x_24 == 0) { -lean_object* x_22; lean_object* x_23; -x_22 = lean_box(0); -x_23 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__5(x_4, x_5, x_3, x_1, x_2, x_22, x_6, x_7, x_8, x_9, x_10); -return x_23; +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_25 = lean_ctor_get(x_22, 0); +x_26 = lean_unsigned_to_nat(0u); +x_27 = l_Array_extract___rarg(x_2, x_26, x_3); +x_28 = l_Lean_mkAppN(x_25, x_27); +lean_dec(x_27); +lean_ctor_set(x_22, 0, x_28); +return x_22; } else { -lean_object* 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_2); -lean_dec(x_1); -x_24 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_24, 0, x_3); -lean_ctor_set(x_24, 1, x_10); -return x_24; +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_22, 0); +lean_inc(x_29); +lean_dec(x_22); +x_30 = lean_unsigned_to_nat(0u); +x_31 = l_Array_extract___rarg(x_2, x_30, x_3); +x_32 = l_Lean_mkAppN(x_29, x_31); +lean_dec(x_31); +x_33 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_33, 0, x_32); +return x_33; } } } } } -LEAN_EXPORT lean_object* l_List_allM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___spec__1___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_8; -x_8 = l_List_allM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -lean_dec(x_2); -return x_8; +lean_object* x_12; lean_object* x_13; uint8_t x_14; uint8_t x_15; uint8_t x_16; lean_object* x_17; +lean_inc(x_3); +x_12 = lean_alloc_closure((void*)(l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___spec__1___lambda__1___boxed), 4, 3); +lean_closure_set(x_12, 0, x_1); +lean_closure_set(x_12, 1, x_3); +lean_closure_set(x_12, 2, x_2); +x_13 = lean_replace_expr(x_12, x_4); +lean_dec(x_12); +x_14 = 0; +x_15 = 1; +x_16 = 1; +x_17 = l_Lean_Meta_mkForallFVars(x_3, x_13, x_14, x_15, x_16, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_17) == 0) +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); +lean_dec(x_17); +x_20 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_19); +return x_20; } +else +{ +uint8_t x_21; +x_21 = !lean_is_exclusive(x_17); +if (x_21 == 0) +{ +return x_17; } -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___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) { -_start: +else { -lean_object* x_9; -x_9 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_1); -return x_9; +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_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_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) { -_start: -{ -lean_object* x_8; -x_8 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_8; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_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) { -_start: -{ -lean_object* x_12; -x_12 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_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); -lean_dec(x_6); -lean_dec(x_3); -lean_dec(x_2); -return x_12; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_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) { -_start: -{ -lean_object* x_13; -x_13 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_7); -return x_13; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -lean_object* x_12; -x_12 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_6); -return x_12; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -lean_object* x_12; -x_12 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_6); -return x_12; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___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_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___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: { -uint8_t x_11; -x_11 = lean_usize_dec_lt(x_4, x_3); -if (x_11 == 0) +if (lean_obj_tag(x_4) == 0) { -lean_object* x_12; +lean_object* x_13; 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_3); lean_dec(x_2); lean_dec(x_1); -x_12 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_12, 0, x_5); -lean_ctor_set(x_12, 1, x_10); -return x_12; +x_13 = l_List_reverse___rarg(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_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_13 = lean_array_uget(x_5, x_4); -x_14 = lean_unsigned_to_nat(0u); -x_15 = lean_array_uset(x_5, x_4, x_14); +uint8_t x_15; +x_15 = !lean_is_exclusive(x_4); +if (x_15 == 0) +{ +lean_object* x_16; uint8_t x_17; +x_16 = lean_ctor_get(x_4, 0); +x_17 = !lean_is_exclusive(x_16); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; lean_object* x_24; +x_18 = lean_ctor_get(x_4, 1); +x_19 = lean_ctor_get(x_16, 0); +x_20 = lean_ctor_get(x_16, 1); +lean_inc(x_2); +x_21 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_21, 0, x_2); +lean_inc(x_1); +lean_inc(x_3); +x_22 = lean_alloc_closure((void*)(l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___spec__1___lambda__2___boxed), 11, 2); +lean_closure_set(x_22, 0, x_3); +lean_closure_set(x_22, 1, x_1); +x_23 = 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); -lean_inc(x_1); -x_16 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask(x_1, x_13, x_2, 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; size_t x_19; size_t x_20; lean_object* x_21; -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_16, 1); -lean_inc(x_18); -lean_dec(x_16); -x_19 = 1; -x_20 = lean_usize_add(x_4, x_19); -x_21 = lean_array_uset(x_15, x_4, x_17); -x_4 = x_20; -x_5 = x_21; -x_10 = x_18; -goto _start; -} -else -{ -uint8_t x_23; -lean_dec(x_15); -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_23 = !lean_is_exclusive(x_16); -if (x_23 == 0) -{ -return x_16; -} -else +x_24 = l_Lean_Meta_forallBoundedTelescope___at_Lean_Elab_Term_addAutoBoundImplicits_x27___spec__2___rarg(x_20, x_21, x_22, x_23, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +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_16, 0); -x_25 = lean_ctor_get(x_16, 1); +lean_object* x_25; lean_object* x_26; +x_25 = lean_ctor_get(x_24, 0); lean_inc(x_25); -lean_inc(x_24); -lean_dec(x_16); -x_26 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_26, 0, x_24); -lean_ctor_set(x_26, 1, x_25); -return x_26; -} -} -} -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__2(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -uint8_t x_10; -x_10 = lean_usize_dec_lt(x_3, x_2); -if (x_10 == 0) +x_26 = lean_ctor_get(x_24, 1); +lean_inc(x_26); +lean_dec(x_24); +lean_ctor_set(x_16, 1, x_25); +lean_ctor_set(x_4, 1, x_5); { -lean_object* x_11; -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -x_11 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_11, 0, x_4); -lean_ctor_set(x_11, 1, x_9); -return x_11; +lean_object* _tmp_3 = x_18; +lean_object* _tmp_4 = x_4; +lean_object* _tmp_11 = x_26; +x_4 = _tmp_3; +x_5 = _tmp_4; +x_12 = _tmp_11; } -else -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_12 = lean_array_uget(x_4, x_3); -x_13 = lean_unsigned_to_nat(0u); -x_14 = lean_array_uset(x_4, x_3, x_13); -x_15 = lean_ctor_get(x_12, 1); -lean_inc(x_15); -lean_dec(x_12); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -x_16 = l___private_Lean_Meta_Basic_0__Lean_Meta_instantiateForallAux(x_1, x_13, x_15, x_5, x_6, x_7, x_8, x_9); -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_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -x_19 = l_Lean_Meta_whnfD(x_17, 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; size_t x_22; size_t 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_inc(x_21); -lean_dec(x_19); -x_22 = 1; -x_23 = lean_usize_add(x_3, x_22); -x_24 = lean_array_uset(x_14, x_3, x_20); -x_3 = x_23; -x_4 = x_24; -x_9 = x_21; goto _start; } else { -uint8_t x_26; -lean_dec(x_14); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -x_26 = !lean_is_exclusive(x_19); -if (x_26 == 0) -{ -return x_19; -} -else -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_19, 0); -x_28 = lean_ctor_get(x_19, 1); -lean_inc(x_28); -lean_inc(x_27); +uint8_t x_28; +lean_free_object(x_16); lean_dec(x_19); -x_29 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_29, 0, x_27); -lean_ctor_set(x_29, 1, x_28); -return x_29; -} -} -} -else -{ -uint8_t x_30; -lean_dec(x_14); +lean_free_object(x_4); +lean_dec(x_18); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -x_30 = !lean_is_exclusive(x_16); -if (x_30 == 0) -{ -return x_16; -} -else -{ -lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_31 = lean_ctor_get(x_16, 0); -x_32 = lean_ctor_get(x_16, 1); -lean_inc(x_32); -lean_inc(x_31); -lean_dec(x_16); -x_33 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_33, 0, x_31); -lean_ctor_set(x_33, 1, x_32); -return x_33; -} -} -} -} -} -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___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: -{ -if (lean_obj_tag(x_2) == 0) -{ -lean_object* x_9; lean_object* x_10; -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -x_9 = l_List_reverse___rarg(x_3); -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_9); -lean_ctor_set(x_10, 1, x_8); -return x_10; -} -else -{ -uint8_t x_11; -x_11 = !lean_is_exclusive(x_2); -if (x_11 == 0) -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_12 = lean_ctor_get(x_2, 0); -x_13 = lean_ctor_get(x_2, 1); -x_14 = lean_ctor_get(x_12, 1); -lean_inc(x_14); -lean_dec(x_12); -x_15 = lean_unsigned_to_nat(0u); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -x_16 = l___private_Lean_Meta_Basic_0__Lean_Meta_instantiateForallAux(x_1, x_15, x_14, 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; -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_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -x_19 = l_Lean_Meta_whnfD(x_17, 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; -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_19, 1); -lean_inc(x_21); -lean_dec(x_19); -lean_ctor_set(x_2, 1, x_3); -lean_ctor_set(x_2, 0, x_20); -{ -lean_object* _tmp_1 = x_13; -lean_object* _tmp_2 = x_2; -lean_object* _tmp_7 = x_21; -x_2 = _tmp_1; -x_3 = _tmp_2; -x_8 = _tmp_7; -} -goto _start; -} -else -{ -uint8_t x_23; -lean_free_object(x_2); -lean_dec(x_13); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_23 = !lean_is_exclusive(x_19); -if (x_23 == 0) -{ -return x_19; -} -else -{ -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_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 -{ -uint8_t x_27; -lean_free_object(x_2); -lean_dec(x_13); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); lean_dec(x_3); -x_27 = !lean_is_exclusive(x_16); -if (x_27 == 0) +lean_dec(x_2); +lean_dec(x_1); +x_28 = !lean_is_exclusive(x_24); +if (x_28 == 0) { -return x_16; +return x_24; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_28 = lean_ctor_get(x_16, 0); -x_29 = lean_ctor_get(x_16, 1); +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_24, 0); +x_30 = lean_ctor_get(x_24, 1); +lean_inc(x_30); lean_inc(x_29); -lean_inc(x_28); -lean_dec(x_16); -x_30 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_30, 0, x_28); -lean_ctor_set(x_30, 1, x_29); -return x_30; +lean_dec(x_24); +x_31 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_31, 0, x_29); +lean_ctor_set(x_31, 1, x_30); +return x_31; } } } else { -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_2, 0); -x_32 = lean_ctor_get(x_2, 1); -lean_inc(x_32); -lean_inc(x_31); -lean_dec(x_2); -x_33 = lean_ctor_get(x_31, 1); +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; lean_object* x_38; +x_32 = lean_ctor_get(x_4, 1); +x_33 = lean_ctor_get(x_16, 0); +x_34 = lean_ctor_get(x_16, 1); +lean_inc(x_34); lean_inc(x_33); -lean_dec(x_31); -x_34 = lean_unsigned_to_nat(0u); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -x_35 = l___private_Lean_Meta_Basic_0__Lean_Meta_instantiateForallAux(x_1, x_34, x_33, x_4, x_5, x_6, x_7, x_8); -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_dec(x_16); +lean_inc(x_2); +x_35 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_35, 0, x_2); +lean_inc(x_1); +lean_inc(x_3); +x_36 = lean_alloc_closure((void*)(l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___spec__1___lambda__2___boxed), 11, 2); +lean_closure_set(x_36, 0, x_3); +lean_closure_set(x_36, 1, x_1); +x_37 = 0; +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -x_38 = l_Lean_Meta_whnfD(x_36, x_4, x_5, x_6, x_7, x_37); +x_38 = l_Lean_Meta_forallBoundedTelescope___at_Lean_Elab_Term_addAutoBoundImplicits_x27___spec__2___rarg(x_34, x_35, x_36, x_37, 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; @@ -25907,23 +26130,37 @@ lean_inc(x_39); x_40 = lean_ctor_get(x_38, 1); lean_inc(x_40); lean_dec(x_38); -x_41 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_41, 0, x_39); -lean_ctor_set(x_41, 1, x_3); -x_2 = x_32; -x_3 = x_41; -x_8 = x_40; +x_41 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_41, 0, x_33); +lean_ctor_set(x_41, 1, x_39); +lean_ctor_set(x_4, 1, x_5); +lean_ctor_set(x_4, 0, x_41); +{ +lean_object* _tmp_3 = x_32; +lean_object* _tmp_4 = x_4; +lean_object* _tmp_11 = x_40; +x_4 = _tmp_3; +x_5 = _tmp_4; +x_12 = _tmp_11; +} goto _start; } else { lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; +lean_dec(x_33); +lean_free_object(x_4); lean_dec(x_32); +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_43 = lean_ctor_get(x_38, 0); lean_inc(x_43); x_44 = lean_ctor_get(x_38, 1); @@ -25946,10605 +26183,18820 @@ lean_ctor_set(x_46, 1, x_44); return x_46; } } +} else { -lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; -lean_dec(x_32); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_47 = lean_ctor_get(x_35, 0); -lean_inc(x_47); -x_48 = lean_ctor_get(x_35, 1); +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; uint8_t x_54; lean_object* x_55; +x_47 = lean_ctor_get(x_4, 0); +x_48 = lean_ctor_get(x_4, 1); lean_inc(x_48); -if (lean_is_exclusive(x_35)) { - lean_ctor_release(x_35, 0); - lean_ctor_release(x_35, 1); - x_49 = x_35; -} else { - lean_dec_ref(x_35); - x_49 = lean_box(0); +lean_inc(x_47); +lean_dec(x_4); +x_49 = lean_ctor_get(x_47, 0); +lean_inc(x_49); +x_50 = lean_ctor_get(x_47, 1); +lean_inc(x_50); +if (lean_is_exclusive(x_47)) { + lean_ctor_release(x_47, 0); + lean_ctor_release(x_47, 1); + x_51 = x_47; +} else { + lean_dec_ref(x_47); + x_51 = lean_box(0); } -if (lean_is_scalar(x_49)) { - x_50 = lean_alloc_ctor(1, 2, 0); +lean_inc(x_2); +x_52 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_52, 0, x_2); +lean_inc(x_1); +lean_inc(x_3); +x_53 = lean_alloc_closure((void*)(l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___spec__1___lambda__2___boxed), 11, 2); +lean_closure_set(x_53, 0, x_3); +lean_closure_set(x_53, 1, x_1); +x_54 = 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_55 = l_Lean_Meta_forallBoundedTelescope___at_Lean_Elab_Term_addAutoBoundImplicits_x27___spec__2___rarg(x_50, x_52, x_53, x_54, 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; +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); +if (lean_is_scalar(x_51)) { + x_58 = lean_alloc_ctor(0, 2, 0); } else { - x_50 = x_49; + x_58 = x_51; } -lean_ctor_set(x_50, 0, x_47); -lean_ctor_set(x_50, 1, x_48); -return x_50; +lean_ctor_set(x_58, 0, x_49); +lean_ctor_set(x_58, 1, x_56); +x_59 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_59, 0, x_58); +lean_ctor_set(x_59, 1, x_5); +x_4 = x_48; +x_5 = x_59; +x_12 = x_57; +goto _start; +} +else +{ +lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; +lean_dec(x_51); +lean_dec(x_49); +lean_dec(x_48); +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_61 = lean_ctor_get(x_55, 0); +lean_inc(x_61); +x_62 = lean_ctor_get(x_55, 1); +lean_inc(x_62); +if (lean_is_exclusive(x_55)) { + lean_ctor_release(x_55, 0); + lean_ctor_release(x_55, 1); + x_63 = x_55; +} else { + lean_dec_ref(x_55); + x_63 = lean_box(0); +} +if (lean_is_scalar(x_63)) { + x_64 = lean_alloc_ctor(1, 2, 0); +} else { + x_64 = x_63; +} +lean_ctor_set(x_64, 0, x_61); +lean_ctor_set(x_64, 1, x_62); +return x_64; } } } } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___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_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -if (lean_obj_tag(x_2) == 0) +if (lean_obj_tag(x_4) == 0) { -lean_object* x_9; lean_object* x_10; +lean_object* x_13; 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_5); -lean_dec(x_4); -x_9 = l_List_reverse___rarg(x_3); -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_9); -lean_ctor_set(x_10, 1, x_8); -return x_10; +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_13 = l_List_reverse___rarg(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 { -uint8_t x_11; -x_11 = !lean_is_exclusive(x_2); -if (x_11 == 0) +uint8_t x_15; +x_15 = !lean_is_exclusive(x_4); +if (x_15 == 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); -x_13 = lean_ctor_get(x_2, 1); -x_14 = lean_ctor_get(x_12, 2); -lean_inc(x_14); -lean_dec(x_12); -x_15 = lean_box(0); +lean_object* x_16; uint8_t x_17; +x_16 = lean_ctor_get(x_4, 0); +x_17 = !lean_is_exclusive(x_16); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_18 = lean_ctor_get(x_4, 1); +x_19 = lean_ctor_get(x_16, 0); +x_20 = lean_ctor_get(x_16, 1); +x_21 = lean_ctor_get(x_16, 2); +x_22 = lean_box(0); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -x_16 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__3(x_1, x_14, x_15, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_16) == 0) +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_23 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___spec__1(x_1, x_2, x_3, x_21, x_22, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_23) == 0) { -lean_object* x_17; lean_object* x_18; -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_2, 1, x_3); -lean_ctor_set(x_2, 0, x_17); +lean_object* x_24; lean_object* x_25; +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_ctor_set(x_16, 2, x_24); +lean_ctor_set(x_4, 1, x_5); { -lean_object* _tmp_1 = x_13; -lean_object* _tmp_2 = x_2; -lean_object* _tmp_7 = x_18; -x_2 = _tmp_1; -x_3 = _tmp_2; -x_8 = _tmp_7; +lean_object* _tmp_3 = x_18; +lean_object* _tmp_4 = x_4; +lean_object* _tmp_11 = x_25; +x_4 = _tmp_3; +x_5 = _tmp_4; +x_12 = _tmp_11; } goto _start; } else { -uint8_t x_20; -lean_free_object(x_2); -lean_dec(x_13); +uint8_t x_27; +lean_free_object(x_16); +lean_dec(x_20); +lean_dec(x_19); +lean_free_object(x_4); +lean_dec(x_18); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); lean_dec(x_3); -x_20 = !lean_is_exclusive(x_16); -if (x_20 == 0) +lean_dec(x_2); +lean_dec(x_1); +x_27 = !lean_is_exclusive(x_23); +if (x_27 == 0) { -return x_16; +return x_23; } 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_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_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_24 = lean_ctor_get(x_2, 0); -x_25 = lean_ctor_get(x_2, 1); -lean_inc(x_25); -lean_inc(x_24); -lean_dec(x_2); -x_26 = lean_ctor_get(x_24, 2); -lean_inc(x_26); -lean_dec(x_24); -x_27 = lean_box(0); +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_31 = lean_ctor_get(x_4, 1); +x_32 = lean_ctor_get(x_16, 0); +x_33 = lean_ctor_get(x_16, 1); +x_34 = lean_ctor_get(x_16, 2); +lean_inc(x_34); +lean_inc(x_33); +lean_inc(x_32); +lean_dec(x_16); +x_35 = lean_box(0); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -x_28 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__3(x_1, x_26, x_27, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_28) == 0) +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_36 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___spec__1(x_1, x_2, x_3, x_34, x_35, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_36) == 0) { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_28, 0); -lean_inc(x_29); -x_30 = lean_ctor_get(x_28, 1); -lean_inc(x_30); -lean_dec(x_28); -x_31 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_31, 0, x_29); -lean_ctor_set(x_31, 1, x_3); -x_2 = x_25; -x_3 = x_31; -x_8 = x_30; +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_36, 0); +lean_inc(x_37); +x_38 = lean_ctor_get(x_36, 1); +lean_inc(x_38); +lean_dec(x_36); +x_39 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_39, 0, x_32); +lean_ctor_set(x_39, 1, x_33); +lean_ctor_set(x_39, 2, x_37); +lean_ctor_set(x_4, 1, x_5); +lean_ctor_set(x_4, 0, x_39); +{ +lean_object* _tmp_3 = x_31; +lean_object* _tmp_4 = x_4; +lean_object* _tmp_11 = x_38; +x_4 = _tmp_3; +x_5 = _tmp_4; +x_12 = _tmp_11; +} goto _start; } else { -lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; -lean_dec(x_25); +lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; +lean_dec(x_33); +lean_dec(x_32); +lean_free_object(x_4); +lean_dec(x_31); +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_33 = lean_ctor_get(x_28, 0); -lean_inc(x_33); -x_34 = lean_ctor_get(x_28, 1); -lean_inc(x_34); -if (lean_is_exclusive(x_28)) { - lean_ctor_release(x_28, 0); - lean_ctor_release(x_28, 1); - x_35 = x_28; +lean_dec(x_2); +lean_dec(x_1); +x_41 = lean_ctor_get(x_36, 0); +lean_inc(x_41); +x_42 = lean_ctor_get(x_36, 1); +lean_inc(x_42); +if (lean_is_exclusive(x_36)) { + lean_ctor_release(x_36, 0); + lean_ctor_release(x_36, 1); + x_43 = x_36; } else { - lean_dec_ref(x_28); - x_35 = lean_box(0); + lean_dec_ref(x_36); + x_43 = lean_box(0); } -if (lean_is_scalar(x_35)) { - x_36 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_43)) { + x_44 = lean_alloc_ctor(1, 2, 0); } else { - x_36 = x_35; -} -lean_ctor_set(x_36, 0, x_33); -lean_ctor_set(x_36, 1, x_34); -return x_36; -} -} + x_44 = x_43; } +lean_ctor_set(x_44, 0, x_41); +lean_ctor_set(x_44, 1, x_42); +return x_44; } } -LEAN_EXPORT lean_object* l_List_bindTR_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__5(lean_object* x_1, lean_object* x_2) { -_start: -{ -if (lean_obj_tag(x_1) == 0) -{ -lean_object* x_3; -x_3 = lean_array_to_list(x_2); -return x_3; } else { -lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_4 = lean_ctor_get(x_1, 0); -lean_inc(x_4); -x_5 = lean_ctor_get(x_1, 1); -lean_inc(x_5); -lean_dec(x_1); -x_6 = l_List_foldl___at_Array_appendList___spec__1___rarg(x_2, x_4); -x_1 = x_5; -x_2 = x_6; -goto _start; +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_45 = lean_ctor_get(x_4, 0); +x_46 = lean_ctor_get(x_4, 1); +lean_inc(x_46); +lean_inc(x_45); +lean_dec(x_4); +x_47 = lean_ctor_get(x_45, 0); +lean_inc(x_47); +x_48 = lean_ctor_get(x_45, 1); +lean_inc(x_48); +x_49 = lean_ctor_get(x_45, 2); +lean_inc(x_49); +if (lean_is_exclusive(x_45)) { + lean_ctor_release(x_45, 0); + lean_ctor_release(x_45, 1); + lean_ctor_release(x_45, 2); + x_50 = x_45; +} else { + lean_dec_ref(x_45); + x_50 = lean_box(0); } +x_51 = lean_box(0); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_52 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___spec__1(x_1, x_2, x_3, x_49, x_51, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_52) == 0) +{ +lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; +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); +if (lean_is_scalar(x_50)) { + x_55 = lean_alloc_ctor(0, 3, 0); +} else { + x_55 = x_50; } +lean_ctor_set(x_55, 0, x_47); +lean_ctor_set(x_55, 1, x_48); +lean_ctor_set(x_55, 2, x_53); +x_56 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_56, 0, x_55); +lean_ctor_set(x_56, 1, x_5); +x_4 = x_46; +x_5 = x_56; +x_12 = x_54; +goto _start; } -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__7(uint8_t 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_unbox(x_6); +lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; +lean_dec(x_50); +lean_dec(x_48); +lean_dec(x_47); +lean_dec(x_46); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); -if (x_7 == 0) -{ -if (x_1 == 0) -{ -uint8_t x_8; -x_8 = 1; -return x_8; +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_58 = lean_ctor_get(x_52, 0); +lean_inc(x_58); +x_59 = lean_ctor_get(x_52, 1); +lean_inc(x_59); +if (lean_is_exclusive(x_52)) { + lean_ctor_release(x_52, 0); + lean_ctor_release(x_52, 1); + x_60 = x_52; +} else { + lean_dec_ref(x_52); + x_60 = lean_box(0); } -else -{ -size_t x_9; size_t x_10; -x_9 = 1; -x_10 = lean_usize_add(x_3, x_9); -x_3 = x_10; -goto _start; +if (lean_is_scalar(x_60)) { + x_61 = lean_alloc_ctor(1, 2, 0); +} else { + x_61 = x_60; } +lean_ctor_set(x_61, 0, x_58); +lean_ctor_set(x_61, 1, x_59); +return x_61; } -else -{ -if (x_1 == 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 +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, 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_16; -x_16 = 0; +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkIndFVar2Const(x_1, x_2, x_3); +x_15 = lean_box(0); +x_16 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___spec__2(x_4, x_5, x_14, x_6, x_15, x_7, x_8, x_9, x_10, x_11, x_12, x_13); return x_16; } } -} -LEAN_EXPORT uint8_t l_Array_contains___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__6(lean_object* x_1, uint8_t x_2) { +LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___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_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_object* x_5; +x_5 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___spec__1___lambda__1(x_1, x_2, x_3, x_4); +lean_dec(x_4); lean_dec(x_3); -x_6 = 0; -return x_6; +lean_dec(x_2); +lean_dec(x_1); +return x_5; } -else +} +LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___spec__1___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: { -size_t x_7; size_t x_8; uint8_t x_9; -x_7 = 0; -x_8 = lean_usize_of_nat(x_3); -lean_dec(x_3); -x_9 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__7(x_2, x_1, x_7, x_8); -return x_9; -} +lean_object* x_12; +x_12 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___spec__1___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_12; } } -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__8(lean_object* x_1, size_t x_2, size_t x_3) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, 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_4; -x_4 = lean_usize_dec_eq(x_2, x_3); -if (x_4 == 0) -{ -lean_object* x_5; uint8_t x_6; uint8_t x_7; -x_5 = lean_array_uget(x_1, x_2); -x_6 = 1; -x_7 = l_Array_contains___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__6(x_5, x_6); -lean_dec(x_5); -if (x_7 == 0) -{ -size_t x_8; size_t x_9; -x_8 = 1; -x_9 = lean_usize_add(x_2, x_8); -x_2 = x_9; -goto _start; -} -else -{ -uint8_t x_11; -x_11 = 1; -return x_11; +lean_object* x_14; +x_14 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts(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_2); +lean_dec(x_1); +return x_14; } } -else +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1() { +_start: { -uint8_t x_12; -x_12 = 0; -return x_12; -} +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; } } -LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1(uint8_t x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -if (lean_obj_tag(x_2) == 0) +if (x_1 == 0) { -lean_object* x_4; -lean_dec(x_1); -x_4 = l_List_reverse___rarg(x_3); -return x_4; +lean_object* x_12; lean_object* x_13; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +x_12 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_11); +return x_13; } else { -uint8_t x_5; -x_5 = !lean_is_exclusive(x_2); -if (x_5 == 0) -{ -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; -x_6 = lean_ctor_get(x_2, 0); -x_7 = lean_ctor_get(x_2, 1); -lean_inc(x_1); -x_8 = lean_apply_1(x_1, x_6); -x_9 = l_Lean_MessageData_ofFormat(x_8); -lean_ctor_set(x_2, 1, x_3); -lean_ctor_set(x_2, 0, x_9); +if (x_2 == 0) { -lean_object* _tmp_1 = x_7; -lean_object* _tmp_2 = x_2; -x_2 = _tmp_1; -x_3 = _tmp_2; -} -goto _start; +lean_object* x_14; lean_object* x_15; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +x_14 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; +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; } 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_2, 0); -x_12 = lean_ctor_get(x_2, 1); -lean_inc(x_12); -lean_inc(x_11); -lean_dec(x_2); -lean_inc(x_1); -x_13 = lean_apply_1(x_1, x_11); -x_14 = l_Lean_MessageData_ofFormat(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_3); -x_2 = x_12; -x_3 = x_15; -goto _start; -} -} -} -} -LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: +uint8_t x_16; lean_object* x_17; +x_16 = 0; +x_17 = l___private_Lean_Meta_Constructions_BRecOn_0__Lean_mkBelowOrIBelow(x_3, x_16, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_17) == 0) { -if (lean_obj_tag(x_3) == 0) +uint8_t x_18; +x_18 = !lean_is_exclusive(x_17); +if (x_18 == 0) { -lean_object* x_5; -lean_dec(x_2); -lean_dec(x_1); -x_5 = l_List_reverse___rarg(x_4); -return x_5; +lean_object* x_19; lean_object* x_20; +x_19 = lean_ctor_get(x_17, 0); +lean_dec(x_19); +x_20 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; +lean_ctor_set(x_17, 0, x_20); +return x_17; } else { -uint8_t x_6; -x_6 = !lean_is_exclusive(x_3); -if (x_6 == 0) -{ -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_7 = lean_ctor_get(x_3, 0); -x_8 = lean_ctor_get(x_3, 1); -lean_inc(x_2); -x_9 = lean_apply_1(x_2, x_7); -lean_inc(x_1); -x_10 = lean_apply_1(x_1, x_9); -x_11 = l_Lean_MessageData_ofFormat(x_10); -lean_ctor_set(x_3, 1, x_4); -lean_ctor_set(x_3, 0, x_11); -{ -lean_object* _tmp_2 = x_8; -lean_object* _tmp_3 = x_3; -x_3 = _tmp_2; -x_4 = _tmp_3; +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_17, 1); +lean_inc(x_21); +lean_dec(x_17); +x_22 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_21); +return x_23; } -goto _start; } 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; -x_13 = lean_ctor_get(x_3, 0); -x_14 = lean_ctor_get(x_3, 1); -lean_inc(x_14); -lean_inc(x_13); -lean_dec(x_3); -lean_inc(x_2); -x_15 = lean_apply_1(x_2, x_13); -lean_inc(x_1); -x_16 = lean_apply_1(x_1, x_15); -x_17 = l_Lean_MessageData_ofFormat(x_16); -x_18 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_18, 0, x_17); -lean_ctor_set(x_18, 1, x_4); -x_3 = x_14; -x_4 = x_18; -goto _start; -} -} -} -} -static lean_object* _init_l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11___closed__1() { -_start: +uint8_t x_24; +x_24 = !lean_is_exclusive(x_17); +if (x_24 == 0) { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("false", 5, 5); -return x_1; -} +return x_17; } -static lean_object* _init_l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11___closed__2() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11___closed__1; -x_2 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_17, 0); +x_26 = lean_ctor_get(x_17, 1); +lean_inc(x_26); +lean_inc(x_25); +lean_dec(x_17); +x_27 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +return x_27; } } -static lean_object* _init_l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11___closed__2; -x_2 = l_Lean_MessageData_ofFormat(x_1); -return x_2; } } -static lean_object* _init_l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11___closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("true", 4, 4); -return x_1; } } -static lean_object* _init_l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11___closed__5() { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__2(uint8_t x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11___closed__4; -x_2 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11___closed__6() { -_start: +if (x_1 == 0) { -lean_object* x_1; lean_object* x_2; -x_1 = l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11___closed__5; -x_2 = l_Lean_MessageData_ofFormat(x_1); -return x_2; -} +lean_object* x_12; lean_object* x_13; +x_12 = lean_box(0); +x_13 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1(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_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11(lean_object* x_1, lean_object* x_2) { -_start: +else { -if (lean_obj_tag(x_1) == 0) +if (x_2 == 0) { -lean_object* x_3; -x_3 = l_List_reverse___rarg(x_2); -return x_3; +lean_object* x_14; lean_object* x_15; +x_14 = lean_box(0); +x_15 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1(x_1, x_2, x_3, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_15; } else { -lean_object* x_4; uint8_t x_5; -x_4 = lean_ctor_get(x_1, 0); -lean_inc(x_4); -x_5 = lean_unbox(x_4); -lean_dec(x_4); -if (x_5 == 0) -{ -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; -x_7 = lean_ctor_get(x_1, 1); -x_8 = lean_ctor_get(x_1, 0); -lean_dec(x_8); -x_9 = l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11___closed__3; -lean_ctor_set(x_1, 1, x_2); -lean_ctor_set(x_1, 0, x_9); +uint8_t x_16; lean_object* x_17; +x_16 = 1; +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_3); +x_17 = l___private_Lean_Meta_Constructions_BRecOn_0__Lean_mkBelowOrIBelow(x_3, x_16, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_17) == 0) { -lean_object* _tmp_0 = x_7; -lean_object* _tmp_1 = x_1; -x_1 = _tmp_0; -x_2 = _tmp_1; -} -goto _start; +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); +lean_dec(x_17); +x_20 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1(x_1, x_2, x_3, x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_19); +lean_dec(x_18); +return x_20; } else { -lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_11 = lean_ctor_get(x_1, 1); -lean_inc(x_11); -lean_dec(x_1); -x_12 = l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11___closed__3; -x_13 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_13, 0, x_12); -lean_ctor_set(x_13, 1, x_2); -x_1 = x_11; -x_2 = x_13; -goto _start; -} +uint8_t x_21; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +x_21 = !lean_is_exclusive(x_17); +if (x_21 == 0) +{ +return x_17; } else { -uint8_t x_15; -x_15 = !lean_is_exclusive(x_1); -if (x_15 == 0) -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_1, 1); -x_17 = lean_ctor_get(x_1, 0); +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_18 = l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11___closed__6; -lean_ctor_set(x_1, 1, x_2); -lean_ctor_set(x_1, 0, x_18); -{ -lean_object* _tmp_0 = x_16; -lean_object* _tmp_1 = x_1; -x_1 = _tmp_0; -x_2 = _tmp_1; -} -goto _start; +x_24 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); +return x_24; } -else -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_1, 1); -lean_inc(x_20); -lean_dec(x_1); -x_21 = l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11___closed__6; -x_22 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_22, 0, x_21); -lean_ctor_set(x_22, 1, x_2); -x_1 = x_20; -x_2 = x_22; -goto _start; } } } } } -LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__12(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__3(uint8_t x_1, uint8_t 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) { _start: { -if (lean_obj_tag(x_1) == 0) +if (x_1 == 0) { -lean_object* x_3; -x_3 = l_List_reverse___rarg(x_2); -return x_3; +lean_object* x_14; lean_object* x_15; +x_14 = lean_box(0); +x_15 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__2(x_1, x_2, x_3, x_14, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +return x_15; } else { -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; lean_object* x_10; -x_5 = lean_ctor_get(x_1, 0); -x_6 = lean_ctor_get(x_1, 1); -x_7 = lean_array_to_list(x_5); -x_8 = lean_box(0); -x_9 = l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11(x_7, x_8); -x_10 = l_Lean_MessageData_ofList(x_9); -lean_ctor_set(x_1, 1, x_2); -lean_ctor_set(x_1, 0, x_10); -{ -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_16; lean_object* x_17; +x_16 = lean_box(0); +x_17 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__2(x_1, x_2, x_3, x_16, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +return x_17; } 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_1, 0); -x_13 = lean_ctor_get(x_1, 1); -lean_inc(x_13); -lean_inc(x_12); -lean_dec(x_1); -x_14 = lean_array_to_list(x_12); -x_15 = lean_box(0); -x_16 = l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11(x_14, x_15); -x_17 = l_Lean_MessageData_ofList(x_16); -x_18 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_18, 0, x_17); -lean_ctor_set(x_18, 1, x_2); -x_1 = x_13; -x_2 = x_18; -goto _start; -} -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__1(lean_object* x_1, size_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: +if (x_5 == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; size_t x_17; lean_object* x_18; -x_13 = lean_array_get_size(x_1); -x_14 = lean_unsigned_to_nat(1u); -lean_inc(x_1); -x_15 = l_Array_toSubarray___rarg(x_1, x_14, x_13); -x_16 = l_Array_ofSubarray___rarg(x_15); -lean_dec(x_15); -x_17 = lean_array_size(x_16); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -x_18 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__2(x_6, x_17, x_2, x_16, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_18) == 0) +lean_object* x_18; lean_object* x_19; +x_18 = lean_box(0); +x_19 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__2(x_1, x_2, x_3, x_18, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +return x_19; +} +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_18, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_18, 1); -lean_inc(x_20); -lean_dec(x_18); -x_21 = lean_array_to_list(x_1); -x_22 = lean_box(0); +lean_object* x_20; +lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); -x_23 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__4(x_6, x_21, x_22, x_8, x_9, x_10, x_11, x_20); -if (lean_obj_tag(x_23) == 0) +lean_inc(x_3); +x_20 = l_Lean_mkNoConfusion(x_3, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_20) == 0) { -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_23, 1); -lean_inc(x_25); -lean_dec(x_23); -x_26 = lean_array_to_list(x_19); -x_27 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__3___closed__1; -x_28 = l_List_bindTR_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__5(x_24, x_27); -x_29 = l_List_appendTR___rarg(x_26, x_28); -x_30 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go(x_3, x_4, x_5, x_7, x_29, x_8, x_9, x_10, x_11, x_25); -return x_30; +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_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__2(x_1, x_2, x_3, x_21, x_7, x_8, x_9, x_10, x_11, x_12, x_22); +lean_dec(x_21); +return x_23; } else { -uint8_t x_31; -lean_dec(x_19); +uint8_t x_24; +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); -x_31 = !lean_is_exclusive(x_23); -if (x_31 == 0) +x_24 = !lean_is_exclusive(x_20); +if (x_24 == 0) { -return x_23; +return x_20; } else { -lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_32 = lean_ctor_get(x_23, 0); -x_33 = lean_ctor_get(x_23, 1); -lean_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; -} -} -} -else -{ -uint8_t x_35; -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_35 = !lean_is_exclusive(x_18); -if (x_35 == 0) -{ -return x_18; +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_20, 0); +x_26 = lean_ctor_get(x_20, 1); +lean_inc(x_26); +lean_inc(x_25); +lean_dec(x_20); +x_27 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +return x_27; } -else -{ -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_18, 0); -x_37 = lean_ctor_get(x_18, 1); -lean_inc(x_37); -lean_inc(x_36); -lean_dec(x_18); -x_38 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -return x_38; } } } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1(uint8_t x_1, uint8_t x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, size_t x_6, size_t x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { -lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; uint8_t x_15; lean_object* x_16; lean_object* x_17; -x_11 = lean_array_get_size(x_1); -x_12 = lean_unsigned_to_nat(0u); -x_13 = lean_nat_dec_lt(x_12, x_11); -lean_dec(x_11); -x_14 = lean_array_get_size(x_2); -x_15 = lean_nat_dec_lt(x_12, x_14); -lean_dec(x_14); -lean_inc(x_3); -x_16 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_16, 0, x_3); -if (x_13 == 0) +uint8_t x_16; +x_16 = lean_usize_dec_lt(x_7, x_6); +if (x_16 == 0) { -lean_object* x_30; lean_object* x_31; -x_30 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; -x_31 = l_outOfBounds___rarg(x_30); -x_17 = x_31; -goto block_29; +lean_object* x_17; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_8); +lean_ctor_set(x_17, 1, x_15); +return x_17; } else { -lean_object* x_32; -x_32 = lean_array_fget(x_1, x_12); -x_17 = x_32; -goto block_29; -} -block_29: +lean_object* x_18; lean_object* x_19; lean_object* x_20; +lean_dec(x_8); +x_18 = lean_array_uget(x_5, x_7); +x_19 = lean_ctor_get(x_18, 4); +lean_inc(x_19); +lean_dec(x_18); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_19); +x_20 = l_mkRecOn(x_19, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_20) == 0) { -lean_object* x_18; lean_object* x_19; -x_18 = lean_box_usize(x_4); -lean_inc(x_2); -x_19 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__1___boxed), 12, 5); -lean_closure_set(x_19, 0, x_2); -lean_closure_set(x_19, 1, x_18); -lean_closure_set(x_19, 2, x_1); -lean_closure_set(x_19, 3, x_17); -lean_closure_set(x_19, 4, x_3); -if (x_15 == 0) +if (x_3 == 0) { -lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; lean_object* x_24; -lean_dec(x_2); -x_20 = l_Lean_instInhabitedInductiveType; -x_21 = l_outOfBounds___rarg(x_20); -x_22 = lean_ctor_get(x_21, 1); -lean_inc(x_22); -lean_dec(x_21); -x_23 = 0; -x_24 = l_Lean_Meta_forallBoundedTelescope___at_Lean_Meta_arrowDomainsN___spec__6___rarg(x_22, x_16, x_19, x_23, x_6, x_7, x_8, x_9, x_10); -return x_24; +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_box(0); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +x_23 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__3(x_3, x_4, x_19, x_1, x_2, x_22, x_9, x_10, x_11, x_12, x_13, x_14, x_21); +if (lean_obj_tag(x_23) == 0) +{ +lean_object* x_24; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +if (lean_obj_tag(x_24) == 0) +{ +uint8_t x_25; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +x_25 = !lean_is_exclusive(x_23); +if (x_25 == 0) +{ +lean_object* x_26; lean_object* x_27; +x_26 = lean_ctor_get(x_23, 0); +lean_dec(x_26); +x_27 = lean_ctor_get(x_24, 0); +lean_inc(x_27); +lean_dec(x_24); +lean_ctor_set(x_23, 0, x_27); +return x_23; } else { -lean_object* x_25; lean_object* x_26; uint8_t x_27; lean_object* x_28; -x_25 = lean_array_fget(x_2, x_12); -lean_dec(x_2); -x_26 = lean_ctor_get(x_25, 1); -lean_inc(x_26); -lean_dec(x_25); -x_27 = 0; -x_28 = l_Lean_Meta_forallBoundedTelescope___at_Lean_Meta_arrowDomainsN___spec__6___rarg(x_26, x_16, x_19, x_27, x_6, x_7, x_8, x_9, x_10); -return x_28; -} -} +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_23, 1); +lean_inc(x_28); +lean_dec(x_23); +x_29 = lean_ctor_get(x_24, 0); +lean_inc(x_29); +lean_dec(x_24); +x_30 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_30, 0, x_29); +lean_ctor_set(x_30, 1, x_28); +return x_30; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_11 = lean_array_get_size(x_1); -x_12 = lean_unsigned_to_nat(0u); -x_13 = lean_nat_dec_lt(x_12, x_11); -if (x_13 == 0) +else { -lean_object* x_14; -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_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_3); -lean_ctor_set(x_14, 1, x_10); -return x_14; +lean_object* x_31; lean_object* x_32; size_t x_33; size_t x_34; +x_31 = lean_ctor_get(x_23, 1); +lean_inc(x_31); +lean_dec(x_23); +x_32 = lean_ctor_get(x_24, 0); +lean_inc(x_32); +lean_dec(x_24); +x_33 = 1; +x_34 = lean_usize_add(x_7, x_33); +x_7 = x_34; +x_8 = x_32; +x_15 = x_31; +goto _start; +} } else { -size_t x_15; uint8_t x_16; -x_15 = lean_usize_of_nat(x_11); +uint8_t x_36; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); lean_dec(x_11); -x_16 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__8(x_1, x_4, x_15); -if (x_16 == 0) +x_36 = !lean_is_exclusive(x_23); +if (x_36 == 0) { -lean_object* x_17; -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_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_3); -lean_ctor_set(x_17, 1, x_10); -return x_17; +return x_23; } else { -lean_object* x_18; lean_object* x_19; -x_18 = lean_box(0); -x_19 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__2(x_1, x_2, x_3, x_4, x_18, x_6, x_7, x_8, x_9, x_10); -return x_19; +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_23, 0); +x_38 = lean_ctor_get(x_23, 1); +lean_inc(x_38); +lean_inc(x_37); +lean_dec(x_23); +x_39 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_39, 0, x_37); +lean_ctor_set(x_39, 1, x_38); +return x_39; } } } +else +{ +lean_object* x_40; lean_object* x_41; +x_40 = lean_ctor_get(x_20, 1); +lean_inc(x_40); +lean_dec(x_20); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_19); +x_41 = l_Lean_mkCasesOn(x_19, x_11, x_12, x_13, x_14, x_40); +if (lean_obj_tag(x_41) == 0) +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_42 = lean_ctor_get(x_41, 0); +lean_inc(x_42); +x_43 = lean_ctor_get(x_41, 1); +lean_inc(x_43); +lean_dec(x_41); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +x_44 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__3(x_3, x_4, x_19, x_1, x_2, x_42, x_9, x_10, x_11, x_12, x_13, x_14, x_43); +lean_dec(x_42); +if (lean_obj_tag(x_44) == 0) +{ +lean_object* x_45; +x_45 = lean_ctor_get(x_44, 0); +lean_inc(x_45); +if (lean_obj_tag(x_45) == 0) +{ +uint8_t x_46; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +x_46 = !lean_is_exclusive(x_44); +if (x_46 == 0) +{ +lean_object* x_47; lean_object* x_48; +x_47 = lean_ctor_get(x_44, 0); +lean_dec(x_47); +x_48 = lean_ctor_get(x_45, 0); +lean_inc(x_48); +lean_dec(x_45); +lean_ctor_set(x_44, 0, x_48); +return x_44; } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__4___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("masks: ", 7, 7); -return x_1; +lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_49 = lean_ctor_get(x_44, 1); +lean_inc(x_49); +lean_dec(x_44); +x_50 = lean_ctor_get(x_45, 0); +lean_inc(x_50); +lean_dec(x_45); +x_51 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_51, 0, x_50); +lean_ctor_set(x_51, 1, x_49); +return x_51; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__4___closed__2() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__4___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +lean_object* x_52; lean_object* x_53; size_t x_54; size_t x_55; +x_52 = lean_ctor_get(x_44, 1); +lean_inc(x_52); +lean_dec(x_44); +x_53 = lean_ctor_get(x_45, 0); +lean_inc(x_53); +lean_dec(x_45); +x_54 = 1; +x_55 = lean_usize_add(x_7, x_54); +x_7 = x_55; +x_8 = x_53; +x_15 = x_52; +goto _start; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -size_t x_10; size_t x_11; lean_object* x_12; -x_10 = lean_array_size(x_1); -x_11 = 0; -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_1); -lean_inc(x_2); -x_12 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__1(x_2, x_3, x_10, x_11, x_1, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_12) == 0) +else { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; -x_13 = lean_ctor_get(x_12, 0); -lean_inc(x_13); -x_14 = lean_ctor_get(x_12, 1); -lean_inc(x_14); +uint8_t x_57; +lean_dec(x_14); +lean_dec(x_13); lean_dec(x_12); -x_15 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__3; -x_16 = l_Lean_isTracingEnabledFor___at_Lean_Meta_processPostponed_loop___spec__1(x_15, x_5, x_6, x_7, x_8, x_14); -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_unbox(x_17); -lean_dec(x_17); -if (x_18 == 0) +lean_dec(x_11); +x_57 = !lean_is_exclusive(x_44); +if (x_57 == 0) { -lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_19 = lean_ctor_get(x_16, 1); -lean_inc(x_19); -lean_dec(x_16); -x_20 = lean_box(0); -x_21 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__3(x_13, x_1, x_2, x_11, x_20, x_5, x_6, x_7, x_8, x_19); -return x_21; +return x_44; } else { -uint8_t x_22; -x_22 = !lean_is_exclusive(x_16); -if (x_22 == 0) +lean_object* x_58; lean_object* x_59; lean_object* x_60; +x_58 = lean_ctor_get(x_44, 0); +x_59 = lean_ctor_get(x_44, 1); +lean_inc(x_59); +lean_inc(x_58); +lean_dec(x_44); +x_60 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_60, 0, x_58); +lean_ctor_set(x_60, 1, x_59); +return x_60; +} +} +} +else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_23 = lean_ctor_get(x_16, 1); -x_24 = lean_ctor_get(x_16, 0); -lean_dec(x_24); -lean_inc(x_13); -x_25 = lean_array_to_list(x_13); -x_26 = lean_box(0); -x_27 = l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__12(x_25, x_26); -x_28 = l_Lean_MessageData_ofList(x_27); -x_29 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__4___closed__2; -lean_ctor_set_tag(x_16, 7); -lean_ctor_set(x_16, 1, x_28); -lean_ctor_set(x_16, 0, x_29); -x_30 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5; -x_31 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_31, 0, x_16); -lean_ctor_set(x_31, 1, x_30); -x_32 = l_Lean_addTrace___at_Lean_Meta_processPostponed_loop___spec__2(x_15, x_31, x_5, x_6, x_7, x_8, x_23); -x_33 = lean_ctor_get(x_32, 0); -lean_inc(x_33); -x_34 = lean_ctor_get(x_32, 1); -lean_inc(x_34); -lean_dec(x_32); -x_35 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__3(x_13, x_1, x_2, x_11, x_33, x_5, x_6, x_7, x_8, x_34); -lean_dec(x_33); -return x_35; +uint8_t x_61; +lean_dec(x_19); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +x_61 = !lean_is_exclusive(x_41); +if (x_61 == 0) +{ +return x_41; } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; -x_36 = lean_ctor_get(x_16, 1); -lean_inc(x_36); -lean_dec(x_16); -lean_inc(x_13); -x_37 = lean_array_to_list(x_13); -x_38 = lean_box(0); -x_39 = l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__12(x_37, x_38); -x_40 = l_Lean_MessageData_ofList(x_39); -x_41 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__4___closed__2; -x_42 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_42, 0, x_41); -lean_ctor_set(x_42, 1, x_40); -x_43 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5; -x_44 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_44, 0, x_42); -lean_ctor_set(x_44, 1, x_43); -x_45 = l_Lean_addTrace___at_Lean_Meta_processPostponed_loop___spec__2(x_15, x_44, x_5, x_6, x_7, x_8, x_36); -x_46 = lean_ctor_get(x_45, 0); -lean_inc(x_46); -x_47 = lean_ctor_get(x_45, 1); -lean_inc(x_47); -lean_dec(x_45); -x_48 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__3(x_13, x_1, x_2, x_11, x_46, x_5, x_6, x_7, x_8, x_47); -lean_dec(x_46); -return x_48; +lean_object* x_62; lean_object* x_63; lean_object* x_64; +x_62 = lean_ctor_get(x_41, 0); +x_63 = lean_ctor_get(x_41, 1); +lean_inc(x_63); +lean_inc(x_62); +lean_dec(x_41); +x_64 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_64, 0, x_62); +lean_ctor_set(x_64, 1, x_63); +return x_64; +} } } } else { -uint8_t x_49; -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_2); -lean_dec(x_1); -x_49 = !lean_is_exclusive(x_12); -if (x_49 == 0) +uint8_t x_65; +lean_dec(x_19); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +x_65 = !lean_is_exclusive(x_20); +if (x_65 == 0) { -return x_12; +return x_20; } else { -lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_50 = lean_ctor_get(x_12, 0); -x_51 = lean_ctor_get(x_12, 1); -lean_inc(x_51); -lean_inc(x_50); -lean_dec(x_12); -x_52 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_52, 0, x_50); -lean_ctor_set(x_52, 1, x_51); -return x_52; -} +lean_object* x_66; lean_object* x_67; lean_object* x_68; +x_66 = lean_ctor_get(x_20, 0); +x_67 = lean_ctor_get(x_20, 1); +lean_inc(x_67); +lean_inc(x_66); +lean_dec(x_20); +x_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; } } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_Elab_Command_inductive_autoPromoteIndices; -return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams(lean_object* x_1, lean_object* x_2, lean_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_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__2___lambda__1(uint8_t x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_9; lean_object* x_10; uint8_t x_11; -x_9 = lean_ctor_get(x_6, 2); -lean_inc(x_9); -x_10 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___closed__1; -x_11 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_9, x_10); -lean_dec(x_9); -if (x_11 == 0) +if (x_1 == 0) { -lean_object* x_12; +lean_object* x_12; lean_object* x_13; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); -x_12 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_12, 0, x_1); -lean_ctor_set(x_12, 1, x_8); -return x_12; +x_12 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_11); +return x_13; } else { -lean_object* x_13; lean_object* x_14; -x_13 = lean_box(0); -x_14 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__4(x_2, x_1, x_3, x_13, x_4, x_5, x_6, x_7, x_8); -return x_14; -} -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___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: +if (x_2 == 0) { -size_t x_11; size_t x_12; lean_object* x_13; -x_11 = lean_unbox_usize(x_3); +lean_object* x_14; lean_object* x_15; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_3); -x_12 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_13 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__1(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); -return x_13; -} +x_14 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; +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_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +else { -size_t x_10; size_t x_11; lean_object* x_12; -x_10 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_11 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_12 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__2(x_1, x_10, x_11, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_1); -return x_12; -} -} -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___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: +uint8_t x_16; lean_object* x_17; +x_16 = 1; +x_17 = l_Lean_mkBRecOnOrBInductionOn(x_3, x_16, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_17) == 0) { -lean_object* x_9; -x_9 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__3(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_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: +uint8_t x_18; +x_18 = !lean_is_exclusive(x_17); +if (x_18 == 0) { -lean_object* x_9; -x_9 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_1); -return x_9; -} +lean_object* x_19; lean_object* x_20; +x_19 = lean_ctor_get(x_17, 0); +lean_dec(x_19); +x_20 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; +lean_ctor_set(x_17, 0, x_20); +return x_17; } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: +else { -uint8_t x_5; size_t x_6; size_t x_7; uint8_t x_8; lean_object* x_9; -x_5 = lean_unbox(x_1); -lean_dec(x_1); -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_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__7(x_5, x_2, x_6, x_7); -lean_dec(x_2); -x_9 = lean_box(x_8); -return x_9; +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_17, 1); +lean_inc(x_21); +lean_dec(x_17); +x_22 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_21); +return x_23; } } -LEAN_EXPORT lean_object* l_Array_contains___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__6___boxed(lean_object* x_1, lean_object* x_2) { -_start: +else { -uint8_t x_3; uint8_t x_4; lean_object* x_5; -x_3 = lean_unbox(x_2); -lean_dec(x_2); -x_4 = l_Array_contains___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__6(x_1, x_3); -lean_dec(x_1); -x_5 = lean_box(x_4); -return x_5; -} -} -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: +uint8_t x_24; +x_24 = !lean_is_exclusive(x_17); +if (x_24 == 0) { -size_t x_4; size_t x_5; uint8_t x_6; lean_object* x_7; -x_4 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_5 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_6 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__8(x_1, x_4, x_5); -lean_dec(x_1); -x_7 = lean_box(x_6); -return x_7; -} +return x_17; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: +else { -size_t x_13; lean_object* x_14; -x_13 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_14 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__1(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_6); -return x_14; +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_17, 0); +x_26 = lean_ctor_get(x_17, 1); +lean_inc(x_26); +lean_inc(x_25); +lean_dec(x_17); +x_27 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +return x_27; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___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: -{ -size_t x_11; lean_object* x_12; -x_11 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_12 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__2(x_1, x_2, x_3, x_11, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_5); -return x_12; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -size_t x_11; lean_object* x_12; -x_11 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_12 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__3(x_1, x_2, x_3, x_11, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_5); -return x_12; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__2(uint8_t x_1, uint8_t 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_10; -x_10 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__4(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; -} +uint8_t x_14; +x_14 = lean_usize_dec_lt(x_5, x_4); +if (x_14 == 0) +{ +lean_object* x_15; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_6); +lean_ctor_set(x_15, 1, x_13); +return x_15; } -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { -_start: +else { -uint8_t x_18; -x_18 = lean_nat_dec_le(x_8, x_7); -if (x_18 == 0) +lean_object* x_16; +lean_dec(x_6); +x_16 = lean_array_uget(x_3, x_5); +if (x_1 == 0) { -lean_object* x_19; uint8_t x_20; -x_19 = lean_unsigned_to_nat(0u); -x_20 = lean_nat_dec_eq(x_6, x_19); -if (x_20 == 0) +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_16, 4); +lean_inc(x_17); +lean_dec(x_16); +x_18 = lean_box(0); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +x_19 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__2___lambda__1(x_1, x_2, x_17, x_18, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_19) == 0) { -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_29; uint8_t x_30; uint8_t x_31; lean_object* x_32; -x_21 = lean_unsigned_to_nat(1u); -x_22 = lean_nat_sub(x_6, x_21); -lean_dec(x_6); -x_29 = lean_array_get_size(x_4); -x_30 = lean_nat_dec_lt(x_7, x_29); -lean_dec(x_29); -x_31 = lean_nat_dec_lt(x_7, x_5); -if (x_30 == 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_109; lean_object* x_110; -x_109 = l_Lean_instInhabitedExpr; -x_110 = l_outOfBounds___rarg(x_109); -x_32 = x_110; -goto block_108; +uint8_t x_21; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +x_21 = !lean_is_exclusive(x_19); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; +x_22 = lean_ctor_get(x_19, 0); +lean_dec(x_22); +x_23 = lean_ctor_get(x_20, 0); +lean_inc(x_23); +lean_dec(x_20); +lean_ctor_set(x_19, 0, x_23); +return x_19; } else { -lean_object* x_111; -x_111 = lean_array_fget(x_4, x_7); -x_32 = x_111; -goto block_108; +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_19, 1); +lean_inc(x_24); +lean_dec(x_19); +x_25 = lean_ctor_get(x_20, 0); +lean_inc(x_25); +lean_dec(x_20); +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; } -block_28: +} +else { -lean_object* x_25; lean_object* x_26; -x_25 = lean_ctor_get(x_23, 0); -lean_inc(x_25); -lean_dec(x_23); -x_26 = lean_nat_add(x_7, x_9); -lean_dec(x_7); -x_6 = x_22; -x_7 = x_26; -x_10 = x_25; -x_17 = x_24; +lean_object* x_27; lean_object* x_28; size_t x_29; size_t x_30; +x_27 = lean_ctor_get(x_19, 1); +lean_inc(x_27); +lean_dec(x_19); +x_28 = lean_ctor_get(x_20, 0); +lean_inc(x_28); +lean_dec(x_20); +x_29 = 1; +x_30 = lean_usize_add(x_5, x_29); +x_5 = x_30; +x_6 = x_28; +x_13 = x_27; goto _start; } -block_108: +} +else { -lean_object* x_33; -if (x_31 == 0) +uint8_t x_32; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +x_32 = !lean_is_exclusive(x_19); +if (x_32 == 0) { -lean_object* x_105; lean_object* x_106; -x_105 = l_Lean_Elab_Command_instInhabitedInductiveView; -x_106 = l_outOfBounds___rarg(x_105); -x_33 = x_106; -goto block_104; +return x_19; } else { -lean_object* x_107; -x_107 = lean_array_fget(x_1, x_7); -x_33 = x_107; -goto block_104; +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_19, 0); +x_34 = lean_ctor_get(x_19, 1); +lean_inc(x_34); +lean_inc(x_33); +lean_dec(x_19); +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +return x_35; } -block_104: +} +} +else { -lean_object* x_34; lean_object* x_35; -x_34 = lean_ctor_get(x_33, 1); -lean_inc(x_34); -lean_dec(x_33); -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_32); -x_35 = l_Lean_Elab_Term_addLocalVarInfo(x_34, x_32, x_11, x_12, x_13, x_14, x_15, x_16, x_17); -if (lean_obj_tag(x_35) == 0) +if (x_2 == 0) { -lean_object* x_36; lean_object* x_37; uint8_t x_38; -x_36 = lean_ctor_get(x_35, 1); +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_16, 4); lean_inc(x_36); -lean_dec(x_35); -x_37 = lean_array_get_size(x_2); -x_38 = lean_nat_dec_lt(x_7, x_37); -lean_dec(x_37); -if (x_38 == 0) -{ -lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; uint8_t x_48; uint8_t x_49; lean_object* x_50; -x_39 = l_Lean_Elab_Command_instInhabitedElabHeaderResult; -x_40 = l_outOfBounds___rarg(x_39); -x_41 = lean_ctor_get(x_40, 4); -lean_inc(x_41); -x_42 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_41, x_11, x_12, x_13, x_14, x_15, x_16, x_36); -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_40, 3); -lean_inc(x_45); -x_46 = l_Lean_Expr_replaceFVars(x_43, x_45, x_3); -lean_dec(x_45); -lean_dec(x_43); -x_47 = 0; -x_48 = 1; -x_49 = 1; -lean_inc(x_3); -x_50 = l_Lean_Meta_mkForallFVars(x_3, x_46, x_47, x_48, x_49, x_13, x_14, x_15, x_16, x_44); -if (lean_obj_tag(x_50) == 0) -{ -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; -x_51 = lean_ctor_get(x_50, 0); -lean_inc(x_51); -x_52 = lean_ctor_get(x_50, 1); -lean_inc(x_52); -lean_dec(x_50); -lean_inc(x_40); -lean_inc(x_3); -lean_inc(x_4); -x_53 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors), 11, 4); -lean_closure_set(x_53, 0, x_4); -lean_closure_set(x_53, 1, x_32); -lean_closure_set(x_53, 2, x_3); -lean_closure_set(x_53, 3, x_40); -lean_inc(x_16); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); +lean_dec(x_16); +x_37 = lean_box(0); lean_inc(x_12); lean_inc(x_11); -x_54 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___rarg(x_3, x_53, x_11, x_12, x_13, x_14, x_15, x_16, x_52); -if (lean_obj_tag(x_54) == 0) +lean_inc(x_10); +lean_inc(x_9); +x_38 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__2___lambda__1(x_1, x_2, x_36, x_37, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_38) == 0) { -lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; -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_40, 0); -lean_inc(x_57); -lean_dec(x_40); -x_58 = lean_ctor_get(x_57, 4); -lean_inc(x_58); -lean_dec(x_57); -x_59 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_59, 0, x_58); -lean_ctor_set(x_59, 1, x_51); -lean_ctor_set(x_59, 2, x_55); -x_60 = lean_array_push(x_10, x_59); -x_61 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_61, 0, x_60); -x_23 = x_61; -x_24 = x_56; -goto block_28; -} -else +lean_object* x_39; +x_39 = lean_ctor_get(x_38, 0); +lean_inc(x_39); +if (lean_obj_tag(x_39) == 0) { -uint8_t x_62; -lean_dec(x_51); -lean_dec(x_40); -lean_dec(x_22); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); +uint8_t x_40; lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); -lean_dec(x_7); -lean_dec(x_4); -lean_dec(x_3); -x_62 = !lean_is_exclusive(x_54); -if (x_62 == 0) +lean_dec(x_9); +x_40 = !lean_is_exclusive(x_38); +if (x_40 == 0) { -return x_54; +lean_object* x_41; lean_object* x_42; +x_41 = lean_ctor_get(x_38, 0); +lean_dec(x_41); +x_42 = lean_ctor_get(x_39, 0); +lean_inc(x_42); +lean_dec(x_39); +lean_ctor_set(x_38, 0, x_42); +return x_38; } else { -lean_object* x_63; lean_object* x_64; lean_object* x_65; -x_63 = lean_ctor_get(x_54, 0); -x_64 = lean_ctor_get(x_54, 1); -lean_inc(x_64); -lean_inc(x_63); -lean_dec(x_54); -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_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_38, 1); +lean_inc(x_43); +lean_dec(x_38); +x_44 = lean_ctor_get(x_39, 0); +lean_inc(x_44); +lean_dec(x_39); +x_45 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_45, 0, x_44); +lean_ctor_set(x_45, 1, x_43); +return x_45; +} } +else +{ +lean_object* x_46; lean_object* x_47; size_t x_48; size_t x_49; +x_46 = lean_ctor_get(x_38, 1); +lean_inc(x_46); +lean_dec(x_38); +x_47 = lean_ctor_get(x_39, 0); +lean_inc(x_47); +lean_dec(x_39); +x_48 = 1; +x_49 = lean_usize_add(x_5, x_48); +x_5 = x_49; +x_6 = x_47; +x_13 = x_46; +goto _start; } } else { -uint8_t x_66; -lean_dec(x_40); -lean_dec(x_32); -lean_dec(x_22); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); +uint8_t x_51; lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); -lean_dec(x_7); -lean_dec(x_4); -lean_dec(x_3); -x_66 = !lean_is_exclusive(x_50); -if (x_66 == 0) +lean_dec(x_9); +x_51 = !lean_is_exclusive(x_38); +if (x_51 == 0) { -return x_50; +return x_38; } else { -lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_67 = lean_ctor_get(x_50, 0); -x_68 = lean_ctor_get(x_50, 1); -lean_inc(x_68); -lean_inc(x_67); -lean_dec(x_50); -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_52; lean_object* x_53; lean_object* x_54; +x_52 = lean_ctor_get(x_38, 0); +x_53 = lean_ctor_get(x_38, 1); +lean_inc(x_53); +lean_inc(x_52); +lean_dec(x_38); +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_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; uint8_t x_78; uint8_t x_79; lean_object* x_80; -x_70 = lean_array_fget(x_2, x_7); -x_71 = lean_ctor_get(x_70, 4); -lean_inc(x_71); -x_72 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_71, x_11, x_12, x_13, x_14, x_15, x_16, x_36); -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_70, 3); -lean_inc(x_75); -x_76 = l_Lean_Expr_replaceFVars(x_73, x_75, x_3); -lean_dec(x_75); -lean_dec(x_73); -x_77 = 0; -x_78 = 1; -x_79 = 1; -lean_inc(x_3); -x_80 = l_Lean_Meta_mkForallFVars(x_3, x_76, x_77, x_78, x_79, x_13, x_14, x_15, x_16, x_74); -if (lean_obj_tag(x_80) == 0) -{ -lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; -x_81 = lean_ctor_get(x_80, 0); -lean_inc(x_81); -x_82 = lean_ctor_get(x_80, 1); -lean_inc(x_82); -lean_dec(x_80); -lean_inc(x_70); -lean_inc(x_3); -lean_inc(x_4); -x_83 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors), 11, 4); -lean_closure_set(x_83, 0, x_4); -lean_closure_set(x_83, 1, x_32); -lean_closure_set(x_83, 2, x_3); -lean_closure_set(x_83, 3, x_70); -lean_inc(x_16); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); +lean_object* x_55; uint8_t x_56; lean_object* x_57; +x_55 = lean_ctor_get(x_16, 4); +lean_inc(x_55); +lean_dec(x_16); +x_56 = 0; lean_inc(x_12); lean_inc(x_11); -x_84 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___rarg(x_3, x_83, x_11, x_12, x_13, x_14, x_15, x_16, x_82); -if (lean_obj_tag(x_84) == 0) +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_55); +x_57 = l_Lean_mkBRecOnOrBInductionOn(x_55, x_56, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_57) == 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; -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_70, 0); -lean_inc(x_87); -lean_dec(x_70); -x_88 = lean_ctor_get(x_87, 4); -lean_inc(x_88); -lean_dec(x_87); -x_89 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_89, 0, x_88); -lean_ctor_set(x_89, 1, x_81); -lean_ctor_set(x_89, 2, x_85); -x_90 = lean_array_push(x_10, x_89); -x_91 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_91, 0, x_90); -x_23 = x_91; -x_24 = x_86; -goto block_28; -} -else +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_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +x_60 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__2___lambda__1(x_1, x_2, x_55, x_58, x_7, x_8, x_9, x_10, x_11, x_12, x_59); +lean_dec(x_58); +if (lean_obj_tag(x_60) == 0) { -uint8_t x_92; -lean_dec(x_81); -lean_dec(x_70); -lean_dec(x_22); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); +lean_object* x_61; +x_61 = lean_ctor_get(x_60, 0); +lean_inc(x_61); +if (lean_obj_tag(x_61) == 0) +{ +uint8_t x_62; lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); -lean_dec(x_7); -lean_dec(x_4); -lean_dec(x_3); -x_92 = !lean_is_exclusive(x_84); -if (x_92 == 0) +lean_dec(x_9); +x_62 = !lean_is_exclusive(x_60); +if (x_62 == 0) { -return x_84; +lean_object* x_63; lean_object* x_64; +x_63 = lean_ctor_get(x_60, 0); +lean_dec(x_63); +x_64 = lean_ctor_get(x_61, 0); +lean_inc(x_64); +lean_dec(x_61); +lean_ctor_set(x_60, 0, x_64); +return x_60; } else { -lean_object* x_93; lean_object* x_94; lean_object* x_95; -x_93 = lean_ctor_get(x_84, 0); -x_94 = lean_ctor_get(x_84, 1); -lean_inc(x_94); -lean_inc(x_93); -lean_dec(x_84); -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_65; lean_object* x_66; lean_object* x_67; +x_65 = lean_ctor_get(x_60, 1); +lean_inc(x_65); +lean_dec(x_60); +x_66 = lean_ctor_get(x_61, 0); +lean_inc(x_66); +lean_dec(x_61); +x_67 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_67, 0, x_66); +lean_ctor_set(x_67, 1, x_65); +return x_67; } } +else +{ +lean_object* x_68; lean_object* x_69; size_t x_70; size_t x_71; +x_68 = lean_ctor_get(x_60, 1); +lean_inc(x_68); +lean_dec(x_60); +x_69 = lean_ctor_get(x_61, 0); +lean_inc(x_69); +lean_dec(x_61); +x_70 = 1; +x_71 = lean_usize_add(x_5, x_70); +x_5 = x_71; +x_6 = x_69; +x_13 = x_68; +goto _start; +} } else { -uint8_t x_96; -lean_dec(x_70); -lean_dec(x_32); -lean_dec(x_22); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); +uint8_t x_73; lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); -lean_dec(x_7); -lean_dec(x_4); -lean_dec(x_3); -x_96 = !lean_is_exclusive(x_80); -if (x_96 == 0) +lean_dec(x_9); +x_73 = !lean_is_exclusive(x_60); +if (x_73 == 0) { -return x_80; +return x_60; } else { -lean_object* x_97; lean_object* x_98; lean_object* x_99; -x_97 = lean_ctor_get(x_80, 0); -x_98 = lean_ctor_get(x_80, 1); -lean_inc(x_98); -lean_inc(x_97); -lean_dec(x_80); -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_74; lean_object* x_75; lean_object* x_76; +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); +x_76 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_76, 0, x_74); +lean_ctor_set(x_76, 1, x_75); +return x_76; } } } else { -uint8_t x_100; -lean_dec(x_32); -lean_dec(x_22); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); +uint8_t x_77; +lean_dec(x_55); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); -lean_dec(x_7); -lean_dec(x_4); -lean_dec(x_3); -x_100 = !lean_is_exclusive(x_35); -if (x_100 == 0) +lean_dec(x_9); +x_77 = !lean_is_exclusive(x_57); +if (x_77 == 0) { -return x_35; +return x_57; } else { -lean_object* x_101; lean_object* x_102; lean_object* x_103; -x_101 = lean_ctor_get(x_35, 0); -x_102 = lean_ctor_get(x_35, 1); -lean_inc(x_102); -lean_inc(x_101); -lean_dec(x_35); -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_78; lean_object* x_79; lean_object* x_80; +x_78 = lean_ctor_get(x_57, 0); +x_79 = lean_ctor_get(x_57, 1); +lean_inc(x_79); +lean_inc(x_78); +lean_dec(x_57); +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 +} +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__1() { +_start: { -lean_object* x_112; -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_7); -lean_dec(x_6); -lean_dec(x_4); -lean_dec(x_3); -x_112 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_112, 0, x_10); -lean_ctor_set(x_112, 1, x_17); -return x_112; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Eq", 2, 2); +return x_1; } } -else +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__2() { +_start: { -lean_object* x_113; -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_7); -lean_dec(x_6); -lean_dec(x_4); -lean_dec(x_3); -x_113 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_113, 0, x_10); -lean_ctor_set(x_113, 1, x_17); -return x_113; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("HEq", 3, 3); +return x_1; +} } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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) { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__4() { _start: { -uint8_t x_14; -x_14 = lean_usize_dec_lt(x_5, x_4); -if (x_14 == 0) +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__3; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__5() { +_start: { -lean_object* x_15; -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_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; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("PUnit", 5, 5); +return x_1; } -else +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__6() { +_start: { -lean_object* x_16; lean_object* x_17; lean_object* x_18; -lean_dec(x_6); -x_16 = lean_array_uget(x_3, x_5); -x_17 = lean_ctor_get(x_16, 2); -lean_inc(x_17); -lean_inc(x_7); -x_18 = l_Lean_mkConstWithLevelParams___at_Lean_Elab_Term_expandDeclId___spec__7(x_17, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_18) == 0) +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__5; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__7() { +_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; uint8_t x_25; lean_object* x_26; -x_19 = lean_ctor_get(x_18, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_18, 1); -lean_inc(x_20); -lean_dec(x_18); -x_21 = lean_ctor_get(x_16, 0); -lean_inc(x_21); -lean_dec(x_16); -x_22 = lean_unsigned_to_nat(3u); -x_23 = l_Lean_Syntax_getArg(x_21, x_22); -lean_dec(x_21); -x_24 = lean_box(0); -x_25 = 1; -lean_inc(x_12); -lean_inc(x_11); +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Prod", 4, 4); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__7; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions(lean_object* x_1, lean_object* x_2, lean_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; lean_object* x_15; uint8_t x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; uint8_t x_20; size_t x_21; size_t x_22; lean_object* x_23; lean_object* x_24; +x_9 = lean_st_ref_get(x_7, x_8); +x_10 = lean_ctor_get(x_9, 0); lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); +x_11 = lean_ctor_get(x_9, 1); +lean_inc(x_11); +lean_dec(x_9); +x_12 = lean_ctor_get(x_10, 0); +lean_inc(x_12); +lean_dec(x_10); +x_13 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__2; +lean_inc(x_12); +x_14 = l_Lean_Environment_contains(x_12, x_13); +x_15 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__4; +lean_inc(x_12); +x_16 = l_Lean_Environment_contains(x_12, x_15); +x_17 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__6; +lean_inc(x_12); +x_18 = l_Lean_Environment_contains(x_12, x_17); +x_19 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___closed__8; +x_20 = l_Lean_Environment_contains(x_12, x_19); +x_21 = lean_array_size(x_1); +x_22 = 0; +x_23 = lean_box(0); lean_inc(x_7); -lean_inc(x_2); -lean_inc(x_1); -x_26 = l_Lean_Elab_Term_addTermInfo_x27(x_23, x_19, x_1, x_2, x_24, x_25, x_7, x_8, x_9, x_10, x_11, x_12, x_20); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_24 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1(x_14, x_16, x_18, x_20, x_1, x_21, x_22, x_23, x_2, x_3, x_4, x_5, x_6, x_7, x_11); +if (lean_obj_tag(x_24) == 0) +{ +lean_object* x_25; lean_object* x_26; +x_25 = lean_ctor_get(x_24, 1); +lean_inc(x_25); +lean_dec(x_24); +x_26 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__2(x_18, x_20, x_1, x_21, x_22, x_23, x_2, x_3, x_4, x_5, x_6, x_7, x_25); if (lean_obj_tag(x_26) == 0) { -lean_object* x_27; size_t x_28; size_t x_29; lean_object* x_30; -x_27 = lean_ctor_get(x_26, 1); -lean_inc(x_27); +uint8_t x_27; +x_27 = !lean_is_exclusive(x_26); +if (x_27 == 0) +{ +lean_object* x_28; +x_28 = lean_ctor_get(x_26, 0); +lean_dec(x_28); +lean_ctor_set(x_26, 0, x_23); +return x_26; +} +else +{ +lean_object* x_29; lean_object* x_30; +x_29 = lean_ctor_get(x_26, 1); +lean_inc(x_29); lean_dec(x_26); -x_28 = 1; -x_29 = lean_usize_add(x_5, x_28); -x_30 = lean_box(0); -x_5 = x_29; -x_6 = x_30; -x_13 = x_27; -goto _start; +x_30 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_30, 0, x_23); +lean_ctor_set(x_30, 1, x_29); +return x_30; +} } else { -uint8_t x_32; -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_2); -lean_dec(x_1); -x_32 = !lean_is_exclusive(x_26); -if (x_32 == 0) +uint8_t x_31; +x_31 = !lean_is_exclusive(x_26); +if (x_31 == 0) { return x_26; } else { -lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_33 = lean_ctor_get(x_26, 0); -x_34 = lean_ctor_get(x_26, 1); -lean_inc(x_34); +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_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_34 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_34, 0, x_32); +lean_ctor_set(x_34, 1, x_33); +return x_34; } } } else { -uint8_t x_36; -lean_dec(x_16); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); +uint8_t x_35; lean_dec(x_7); -lean_dec(x_2); -lean_dec(x_1); -x_36 = !lean_is_exclusive(x_18); -if (x_36 == 0) +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_35 = !lean_is_exclusive(x_24); +if (x_35 == 0) { -return x_18; +return x_24; } else { -lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_37 = lean_ctor_get(x_18, 0); -x_38 = lean_ctor_get(x_18, 1); -lean_inc(x_38); +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_24, 0); +x_37 = lean_ctor_get(x_24, 1); lean_inc(x_37); -lean_dec(x_18); -x_39 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_39, 0, x_37); -lean_ctor_set(x_39, 1, x_38); -return x_39; -} +lean_inc(x_36); +lean_dec(x_24); +x_38 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_38, 0, x_36); +lean_ctor_set(x_38, 1, x_37); +return x_38; } } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -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); +uint8_t x_12; uint8_t x_13; lean_object* x_14; +x_12 = lean_unbox(x_1); +lean_dec(x_1); +x_13 = lean_unbox(x_2); +lean_dec(x_2); +x_14 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1(x_12, x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_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; +lean_dec(x_4); +return x_14; } -else +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: { -lean_object* x_14; lean_object* x_15; lean_object* x_16; +uint8_t x_12; uint8_t x_13; lean_object* x_14; +x_12 = lean_unbox(x_1); +lean_dec(x_1); +x_13 = lean_unbox(x_2); +lean_dec(x_2); +x_14 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__2(x_12, x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); -x_14 = lean_array_uget(x_1, x_3); -x_15 = lean_ctor_get(x_14, 4); -lean_inc(x_15); -lean_inc(x_5); -lean_inc(x_15); -x_16 = l_Lean_mkConstWithLevelParams___at_Lean_Elab_Term_expandDeclId___spec__7(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; uint8_t x_24; lean_object* x_25; -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_16, 1); -lean_inc(x_18); -lean_dec(x_16); -x_19 = lean_ctor_get(x_14, 0); -lean_inc(x_19); -x_20 = lean_unsigned_to_nat(1u); -x_21 = l_Lean_Syntax_getArg(x_19, x_20); -lean_dec(x_19); -x_22 = lean_box(0); -x_23 = lean_box(0); -x_24 = 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_25 = l_Lean_Elab_Term_addTermInfo_x27(x_21, x_17, x_22, x_22, x_23, x_24, x_5, x_6, x_7, x_8, x_9, x_10, x_18); -if (lean_obj_tag(x_25) == 0) -{ -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_26 = lean_ctor_get(x_25, 1); -lean_inc(x_26); -lean_dec(x_25); -x_27 = lean_ctor_get(x_14, 8); -lean_inc(x_27); -x_28 = lean_array_size(x_27); -x_29 = 0; -x_30 = 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_31 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__2(x_22, x_22, x_27, x_28, x_29, x_30, x_5, x_6, x_7, x_8, x_9, x_10, x_26); -lean_dec(x_27); -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; -x_32 = lean_ctor_get(x_31, 1); -lean_inc(x_32); -lean_dec(x_31); -x_33 = lean_ctor_get(x_14, 2); -lean_inc(x_33); -lean_dec(x_14); -x_34 = lean_ctor_get(x_33, 1); -lean_inc(x_34); -lean_dec(x_33); -x_35 = 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_36 = l_Lean_Elab_Term_applyAttributesAt(x_15, x_34, x_35, x_5, x_6, x_7, x_8, x_9, x_10, x_32); -if (lean_obj_tag(x_36) == 0) -{ -lean_object* x_37; size_t x_38; size_t x_39; -x_37 = lean_ctor_get(x_36, 1); -lean_inc(x_37); -lean_dec(x_36); -x_38 = 1; -x_39 = lean_usize_add(x_3, x_38); -x_3 = x_39; -x_4 = x_30; -x_11 = x_37; -goto _start; +return x_14; } -else +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: { -uint8_t x_41; -lean_dec(x_10); -lean_dec(x_9); +uint8_t x_14; uint8_t x_15; uint8_t x_16; uint8_t x_17; lean_object* x_18; +x_14 = lean_unbox(x_1); +lean_dec(x_1); +x_15 = lean_unbox(x_2); +lean_dec(x_2); +x_16 = lean_unbox(x_4); +lean_dec(x_4); +x_17 = lean_unbox(x_5); +lean_dec(x_5); +x_18 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__3(x_14, x_15, x_3, x_16, x_17, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -x_41 = !lean_is_exclusive(x_36); -if (x_41 == 0) -{ -return x_36; -} -else -{ -lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_ctor_get(x_36, 0); -x_43 = lean_ctor_get(x_36, 1); -lean_inc(x_43); -lean_inc(x_42); -lean_dec(x_36); -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; -} +return x_18; } } -else +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +_start: { -uint8_t x_45; -lean_dec(x_15); -lean_dec(x_14); +uint8_t x_16; uint8_t x_17; uint8_t x_18; uint8_t x_19; size_t x_20; size_t x_21; lean_object* x_22; +x_16 = lean_unbox(x_1); +lean_dec(x_1); +x_17 = lean_unbox(x_2); +lean_dec(x_2); +x_18 = lean_unbox(x_3); +lean_dec(x_3); +x_19 = lean_unbox(x_4); +lean_dec(x_4); +x_20 = lean_unbox_usize(x_6); +lean_dec(x_6); +x_21 = lean_unbox_usize(x_7); +lean_dec(x_7); +x_22 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1(x_16, x_17, x_18, x_19, x_5, x_20, x_21, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); lean_dec(x_5); -x_45 = !lean_is_exclusive(x_31); -if (x_45 == 0) -{ -return x_31; -} -else -{ -lean_object* x_46; lean_object* x_47; lean_object* x_48; -x_46 = lean_ctor_get(x_31, 0); -x_47 = lean_ctor_get(x_31, 1); -lean_inc(x_47); -lean_inc(x_46); -lean_dec(x_31); -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; -} +return x_22; } } -else +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___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: { -uint8_t x_49; -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); +uint8_t x_12; uint8_t x_13; lean_object* x_14; +x_12 = lean_unbox(x_1); +lean_dec(x_1); +x_13 = lean_unbox(x_2); +lean_dec(x_2); +x_14 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__2___lambda__1(x_12, x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_6); lean_dec(x_5); -x_49 = !lean_is_exclusive(x_25); -if (x_49 == 0) -{ -return x_25; -} -else -{ -lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_50 = lean_ctor_get(x_25, 0); -x_51 = lean_ctor_get(x_25, 1); -lean_inc(x_51); -lean_inc(x_50); -lean_dec(x_25); -x_52 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_52, 0, x_50); -lean_ctor_set(x_52, 1, x_51); -return x_52; -} +lean_dec(x_4); +return x_14; } } -else +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: { -uint8_t x_53; -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_10); -lean_dec(x_9); +uint8_t x_14; uint8_t x_15; size_t x_16; size_t x_17; lean_object* x_18; +x_14 = lean_unbox(x_1); +lean_dec(x_1); +x_15 = lean_unbox(x_2); +lean_dec(x_2); +x_16 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_17 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_18 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__2(x_14, x_15, x_3, x_16, x_17, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -x_53 = !lean_is_exclusive(x_16); -if (x_53 == 0) -{ -return x_16; +lean_dec(x_3); +return x_18; } -else -{ -lean_object* x_54; lean_object* x_55; lean_object* x_56; -x_54 = lean_ctor_get(x_16, 0); -x_55 = lean_ctor_get(x_16, 1); -lean_inc(x_55); -lean_inc(x_54); -lean_dec(x_16); -x_56 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_56, 0, x_54); -lean_ctor_set(x_56, 1, x_55); -return x_56; } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___boxed(lean_object* x_1, lean_object* x_2, lean_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_Inductive_0__Lean_Elab_Command_mkAuxConstructions(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_Elab_Inductive_0__Lean_Elab_Command_getArity___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; lean_object* x_9; +x_8 = lean_array_get_size(x_1); +x_9 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_9, 0, x_8); +lean_ctor_set(x_9, 1, x_7); +return x_9; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__8(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) { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getArity___closed__1() { _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_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_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getArity___lambda__1___boxed), 7, 0); +return x_1; } -else +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getArity(lean_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_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_object* x_7; lean_object* x_8; uint8_t x_9; lean_object* x_10; +x_7 = lean_ctor_get(x_1, 1); lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_2); -lean_inc(x_1); -x_18 = l_Lean_PersistentArray_mapMAux___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__7(x_1, x_2, x_15, 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; 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_4, x_21); -x_23 = lean_array_uset(x_17, x_4, x_19); -x_4 = x_22; -x_5 = x_23; -x_12 = x_20; -goto _start; +lean_dec(x_1); +x_8 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getArity___closed__1; +x_9 = 0; +x_10 = l_Lean_Meta_forallTelescopeReducing___at_Lean_Meta_getParamNames___spec__2___rarg(x_7, x_8, x_9, x_2, x_3, x_4, x_5, x_6); +return x_10; } -else +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getArity___lambda__1___boxed(lean_object* x_1, 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_25; -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_object* x_8; +x_8 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getArity___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_25 = !lean_is_exclusive(x_18); -if (x_25 == 0) +return x_8; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_resetMaskAt(lean_object* x_1, lean_object* x_2) { +_start: { -return x_18; +lean_object* x_3; uint8_t x_4; +x_3 = lean_array_get_size(x_1); +x_4 = lean_nat_dec_lt(x_2, x_3); +lean_dec(x_3); +if (x_4 == 0) +{ +return x_1; } 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; +uint8_t x_5; lean_object* x_6; lean_object* x_7; +x_5 = 0; +x_6 = lean_box(x_5); +x_7 = lean_array_fset(x_1, x_2, x_6); +return x_7; } } } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_resetMaskAt___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_resetMaskAt(x_1, x_2); +lean_dec(x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__9(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_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -uint8_t x_13; -x_13 = lean_usize_dec_lt(x_4, x_3); -if (x_13 == 0) +uint8_t x_14; +x_14 = lean_nat_dec_le(x_6, x_5); +if (x_14 == 0) { -lean_object* x_14; -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); +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_36; uint8_t x_37; lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -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; +x_17 = lean_unsigned_to_nat(1u); +x_18 = lean_nat_sub(x_4, x_17); +lean_dec(x_4); +x_36 = lean_array_get_size(x_2); +x_37 = lean_nat_dec_lt(x_5, x_36); +lean_dec(x_36); +if (x_37 == 0) +{ +lean_object* x_38; +x_38 = lean_box(0); +x_25 = x_38; +goto block_35; } 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_array_uget(x_5, x_4); -x_16 = lean_unsigned_to_nat(0u); -x_17 = lean_array_uset(x_5, x_4, x_16); -x_18 = lean_ctor_get(x_2, 0); -lean_inc(x_18); -x_19 = l_Lean_Elab_InfoTree_substitute(x_15, x_18); -lean_inc(x_1); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -x_20 = lean_apply_7(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_20) == 0) +lean_object* x_39; uint8_t x_40; lean_object* x_41; +x_39 = lean_array_get_size(x_3); +x_40 = lean_nat_dec_lt(x_5, x_39); +lean_dec(x_39); +x_41 = lean_array_fget(x_2, x_5); +if (x_40 == 0) { -lean_object* x_21; -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -if (lean_obj_tag(x_21) == 0) +lean_object* x_42; lean_object* x_43; uint8_t x_44; +x_42 = l_Lean_instInhabitedExpr; +x_43 = l_outOfBounds___rarg(x_42); +x_44 = lean_expr_eqv(x_41, x_43); +lean_dec(x_43); +lean_dec(x_41); +if (x_44 == 0) { -lean_object* x_22; size_t x_23; size_t x_24; lean_object* x_25; -x_22 = lean_ctor_get(x_20, 1); -lean_inc(x_22); -lean_dec(x_20); -x_23 = 1; -x_24 = lean_usize_add(x_4, x_23); -x_25 = lean_array_uset(x_17, x_4, x_19); -x_4 = x_24; -x_5 = x_25; -x_12 = x_22; -goto _start; +lean_object* x_45; +x_45 = lean_box(0); +x_25 = x_45; +goto block_35; } else { -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_20, 1); -lean_inc(x_27); -lean_dec(x_20); -x_28 = lean_ctor_get(x_21, 0); -lean_inc(x_28); -lean_dec(x_21); -x_29 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_29, 0, x_28); -lean_ctor_set(x_29, 1, x_19); -x_30 = 1; -x_31 = lean_usize_add(x_4, x_30); -x_32 = lean_array_uset(x_17, x_4, x_29); -x_4 = x_31; -x_5 = x_32; -x_12 = x_27; -goto _start; +lean_object* x_46; +x_46 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; +x_19 = x_46; +x_20 = x_13; +goto block_24; } } else { -uint8_t x_34; -lean_dec(x_19); -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_2); -lean_dec(x_1); -x_34 = !lean_is_exclusive(x_20); -if (x_34 == 0) +lean_object* x_47; uint8_t x_48; +x_47 = lean_array_fget(x_3, x_5); +x_48 = lean_expr_eqv(x_41, x_47); +lean_dec(x_47); +lean_dec(x_41); +if (x_48 == 0) { -return x_20; +lean_object* x_49; +x_49 = lean_box(0); +x_25 = x_49; +goto block_35; } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; -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_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_50; +x_50 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; +x_19 = x_50; +x_20 = x_13; +goto block_24; } } } -LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapMAux___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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: -{ -if (lean_obj_tag(x_3) == 0) +block_24: { -uint8_t x_11; -x_11 = !lean_is_exclusive(x_3); -if (x_11 == 0) -{ -lean_object* x_12; size_t x_13; size_t x_14; lean_object* x_15; -x_12 = lean_ctor_get(x_3, 0); -x_13 = lean_array_size(x_12); -x_14 = 0; -x_15 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__8(x_1, x_2, x_13, x_14, x_12, 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; -x_16 = !lean_is_exclusive(x_15); -if (x_16 == 0) -{ -lean_object* x_17; -x_17 = lean_ctor_get(x_15, 0); -lean_ctor_set(x_3, 0, x_17); -lean_ctor_set(x_15, 0, x_3); -return x_15; +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; } -else +block_35: { -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_15, 0); -x_19 = lean_ctor_get(x_15, 1); -lean_inc(x_19); -lean_inc(x_18); -lean_dec(x_15); -lean_ctor_set(x_3, 0, x_18); -x_20 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_20, 0, x_3); -lean_ctor_set(x_20, 1, x_19); -return x_20; +lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +lean_dec(x_25); +x_26 = lean_st_ref_take(x_1, 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 = 0; +x_30 = lean_box(x_29); +x_31 = lean_array_set(x_27, x_5, x_30); +x_32 = lean_st_ref_set(x_1, x_31, x_28); +x_33 = lean_ctor_get(x_32, 1); +lean_inc(x_33); +lean_dec(x_32); +x_34 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; +x_19 = x_34; +x_20 = x_33; +goto block_24; } } else { -uint8_t x_21; -lean_free_object(x_3); -x_21 = !lean_is_exclusive(x_15); -if (x_21 == 0) -{ -return x_15; +lean_object* x_51; +lean_dec(x_5); +lean_dec(x_4); +x_51 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_51, 0, x_8); +lean_ctor_set(x_51, 1, x_13); +return x_51; +} } else { -lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_22 = lean_ctor_get(x_15, 0); -x_23 = lean_ctor_get(x_15, 1); -lean_inc(x_23); -lean_inc(x_22); -lean_dec(x_15); -x_24 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_24, 0, x_22); -lean_ctor_set(x_24, 1, x_23); -return x_24; +lean_object* x_52; +lean_dec(x_5); +lean_dec(x_4); +x_52 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_52, 0, x_8); +lean_ctor_set(x_52, 1, x_13); +return x_52; } } } -else +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__2(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4) { +_start: { -lean_object* x_25; size_t x_26; size_t x_27; lean_object* x_28; -x_25 = lean_ctor_get(x_3, 0); -lean_inc(x_25); -lean_dec(x_3); -x_26 = lean_array_size(x_25); -x_27 = 0; -x_28 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__8(x_1, x_2, x_26, x_27, x_25, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_28) == 0) +uint8_t x_5; +x_5 = lean_usize_dec_eq(x_3, x_4); +if (x_5 == 0) { -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_29 = lean_ctor_get(x_28, 0); -lean_inc(x_29); -x_30 = lean_ctor_get(x_28, 1); -lean_inc(x_30); -if (lean_is_exclusive(x_28)) { - lean_ctor_release(x_28, 0); - lean_ctor_release(x_28, 1); - x_31 = x_28; -} else { - lean_dec_ref(x_28); - x_31 = lean_box(0); -} -x_32 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_32, 0, x_29); -if (lean_is_scalar(x_31)) { - x_33 = lean_alloc_ctor(0, 2, 0); -} else { - x_33 = x_31; -} -lean_ctor_set(x_33, 0, x_32); -lean_ctor_set(x_33, 1, x_30); -return x_33; +lean_object* x_6; lean_object* x_7; uint8_t x_8; +x_6 = lean_array_uget(x_2, x_3); +x_7 = l_Lean_Expr_getAppFn(x_1); +x_8 = lean_expr_eqv(x_7, x_6); +lean_dec(x_6); +lean_dec(x_7); +if (x_8 == 0) +{ +size_t x_9; size_t x_10; +x_9 = 1; +x_10 = lean_usize_add(x_3, x_9); +x_3 = x_10; +goto _start; } else { -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_34 = lean_ctor_get(x_28, 0); -lean_inc(x_34); -x_35 = lean_ctor_get(x_28, 1); -lean_inc(x_35); -if (lean_is_exclusive(x_28)) { - lean_ctor_release(x_28, 0); - lean_ctor_release(x_28, 1); - x_36 = x_28; -} else { - lean_dec_ref(x_28); - x_36 = lean_box(0); +uint8_t x_12; +x_12 = 1; +return x_12; } -if (lean_is_scalar(x_36)) { - x_37 = lean_alloc_ctor(1, 2, 0); -} else { - x_37 = x_36; } -lean_ctor_set(x_37, 0, x_34); -lean_ctor_set(x_37, 1, x_35); -return x_37; +else +{ +uint8_t x_13; +x_13 = 0; +return x_13; } } } -else +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___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) { +_start: { -uint8_t x_38; -x_38 = !lean_is_exclusive(x_3); -if (x_38 == 0) +uint8_t x_15; +x_15 = lean_nat_dec_le(x_7, x_6); +if (x_15 == 0) { -lean_object* x_39; size_t x_40; size_t x_41; lean_object* x_42; -x_39 = lean_ctor_get(x_3, 0); -x_40 = lean_array_size(x_39); -x_41 = 0; -x_42 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__9(x_1, x_2, x_40, x_41, x_39, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_42) == 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) { -uint8_t x_43; -x_43 = !lean_is_exclusive(x_42); -if (x_43 == 0) +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_27; uint8_t x_28; +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_27 = lean_array_get_size(x_2); +x_28 = lean_nat_dec_le(x_27, x_6); +if (x_28 == 0) { -lean_object* x_44; -x_44 = lean_ctor_get(x_42, 0); -lean_ctor_set(x_3, 0, x_44); -lean_ctor_set(x_42, 0, x_3); -return x_42; -} -else +uint8_t x_29; uint8_t x_30; +x_29 = lean_nat_dec_lt(x_6, x_4); +x_30 = lean_nat_dec_lt(x_6, x_27); +lean_dec(x_27); +if (x_29 == 0) { -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_42, 0); -x_46 = lean_ctor_get(x_42, 1); -lean_inc(x_46); -lean_inc(x_45); -lean_dec(x_42); -lean_ctor_set(x_3, 0, x_45); -x_47 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_47, 0, x_3); -lean_ctor_set(x_47, 1, x_46); -return x_47; -} -} -else +lean_object* x_31; lean_object* x_32; +x_31 = l_Lean_instInhabitedExpr; +x_32 = l_outOfBounds___rarg(x_31); +if (x_30 == 0) { -uint8_t x_48; -lean_free_object(x_3); -x_48 = !lean_is_exclusive(x_42); -if (x_48 == 0) +lean_object* x_33; uint8_t x_34; +x_33 = l_outOfBounds___rarg(x_31); +x_34 = lean_expr_eqv(x_32, x_33); +lean_dec(x_33); +lean_dec(x_32); +if (x_34 == 0) { -return x_42; +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; +x_35 = lean_st_ref_take(x_1, x_14); +x_36 = lean_ctor_get(x_35, 0); +lean_inc(x_36); +x_37 = lean_ctor_get(x_35, 1); +lean_inc(x_37); +lean_dec(x_35); +x_38 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_resetMaskAt(x_36, x_6); +x_39 = lean_st_ref_set(x_1, x_38, x_37); +x_40 = !lean_is_exclusive(x_39); +if (x_40 == 0) +{ +lean_object* x_41; lean_object* x_42; +x_41 = lean_ctor_get(x_39, 0); +lean_dec(x_41); +x_42 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; +lean_ctor_set(x_39, 0, x_42); +x_20 = x_39; +goto block_26; } else { -lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_49 = lean_ctor_get(x_42, 0); -x_50 = lean_ctor_get(x_42, 1); -lean_inc(x_50); -lean_inc(x_49); -lean_dec(x_42); -x_51 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_51, 0, x_49); -lean_ctor_set(x_51, 1, x_50); -return x_51; +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_39, 1); +lean_inc(x_43); +lean_dec(x_39); +x_44 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; +x_45 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_45, 0, x_44); +lean_ctor_set(x_45, 1, x_43); +x_20 = x_45; +goto block_26; +} } +else +{ +lean_object* x_46; lean_object* x_47; +x_46 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; +x_47 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_47, 0, x_46); +lean_ctor_set(x_47, 1, x_14); +x_20 = x_47; +goto block_26; } } else { -lean_object* x_52; size_t x_53; size_t x_54; lean_object* x_55; -x_52 = lean_ctor_get(x_3, 0); +lean_object* x_48; uint8_t x_49; +x_48 = lean_array_fget(x_2, x_6); +x_49 = lean_expr_eqv(x_32, x_48); +lean_dec(x_48); +lean_dec(x_32); +if (x_49 == 0) +{ +lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; uint8_t x_55; +x_50 = lean_st_ref_take(x_1, x_14); +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_3); -x_53 = lean_array_size(x_52); -x_54 = 0; -x_55 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__9(x_1, x_2, x_53, x_54, x_52, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_55) == 0) +lean_dec(x_50); +x_53 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_resetMaskAt(x_51, x_6); +x_54 = lean_st_ref_set(x_1, x_53, x_52); +x_55 = !lean_is_exclusive(x_54); +if (x_55 == 0) { -lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_56 = lean_ctor_get(x_55, 0); -lean_inc(x_56); -x_57 = lean_ctor_get(x_55, 1); -lean_inc(x_57); -if (lean_is_exclusive(x_55)) { - lean_ctor_release(x_55, 0); - lean_ctor_release(x_55, 1); - x_58 = x_55; -} else { - lean_dec_ref(x_55); - x_58 = lean_box(0); -} -x_59 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_59, 0, x_56); -if (lean_is_scalar(x_58)) { - x_60 = lean_alloc_ctor(0, 2, 0); -} else { - x_60 = x_58; -} -lean_ctor_set(x_60, 0, x_59); -lean_ctor_set(x_60, 1, x_57); -return x_60; +lean_object* x_56; lean_object* x_57; +x_56 = lean_ctor_get(x_54, 0); +lean_dec(x_56); +x_57 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; +lean_ctor_set(x_54, 0, x_57); +x_20 = x_54; +goto block_26; } else { -lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; -x_61 = lean_ctor_get(x_55, 0); -lean_inc(x_61); -x_62 = lean_ctor_get(x_55, 1); -lean_inc(x_62); -if (lean_is_exclusive(x_55)) { - lean_ctor_release(x_55, 0); - lean_ctor_release(x_55, 1); - x_63 = x_55; -} else { - lean_dec_ref(x_55); - x_63 = lean_box(0); -} -if (lean_is_scalar(x_63)) { - x_64 = lean_alloc_ctor(1, 2, 0); -} else { - x_64 = x_63; -} -lean_ctor_set(x_64, 0, x_61); -lean_ctor_set(x_64, 1, x_62); -return x_64; +lean_object* x_58; lean_object* x_59; lean_object* x_60; +x_58 = lean_ctor_get(x_54, 1); +lean_inc(x_58); +lean_dec(x_54); +x_59 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; +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_20 = x_60; +goto block_26; } } +else +{ +lean_object* x_61; lean_object* x_62; +x_61 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; +x_62 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_62, 0, x_61); +lean_ctor_set(x_62, 1, x_14); +x_20 = x_62; +goto block_26; } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__10(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: +else { -uint8_t x_13; -x_13 = lean_usize_dec_lt(x_4, x_3); -if (x_13 == 0) +lean_object* x_63; +x_63 = lean_array_fget(x_3, x_6); +if (x_30 == 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_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_64; lean_object* x_65; uint8_t x_66; +x_64 = l_Lean_instInhabitedExpr; +x_65 = l_outOfBounds___rarg(x_64); +x_66 = lean_expr_eqv(x_63, x_65); +lean_dec(x_65); +lean_dec(x_63); +if (x_66 == 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_array_uget(x_5, x_4); -x_16 = lean_unsigned_to_nat(0u); -x_17 = lean_array_uset(x_5, x_4, x_16); -x_18 = lean_ctor_get(x_2, 0); -lean_inc(x_18); -x_19 = l_Lean_Elab_InfoTree_substitute(x_15, x_18); -lean_inc(x_1); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -x_20 = lean_apply_7(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_20) == 0) +lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; uint8_t x_72; +x_67 = lean_st_ref_take(x_1, x_14); +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 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_resetMaskAt(x_68, x_6); +x_71 = lean_st_ref_set(x_1, x_70, x_69); +x_72 = !lean_is_exclusive(x_71); +if (x_72 == 0) { -lean_object* x_21; -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -if (lean_obj_tag(x_21) == 0) +lean_object* x_73; lean_object* x_74; +x_73 = lean_ctor_get(x_71, 0); +lean_dec(x_73); +x_74 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; +lean_ctor_set(x_71, 0, x_74); +x_20 = x_71; +goto block_26; +} +else { -lean_object* x_22; size_t x_23; size_t x_24; lean_object* x_25; -x_22 = lean_ctor_get(x_20, 1); -lean_inc(x_22); -lean_dec(x_20); -x_23 = 1; -x_24 = lean_usize_add(x_4, x_23); -x_25 = lean_array_uset(x_17, x_4, x_19); -x_4 = x_24; -x_5 = x_25; -x_12 = x_22; -goto _start; +lean_object* x_75; lean_object* x_76; lean_object* x_77; +x_75 = lean_ctor_get(x_71, 1); +lean_inc(x_75); +lean_dec(x_71); +x_76 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; +x_77 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_77, 0, x_76); +lean_ctor_set(x_77, 1, x_75); +x_20 = x_77; +goto block_26; +} } else { -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_20, 1); -lean_inc(x_27); -lean_dec(x_20); -x_28 = lean_ctor_get(x_21, 0); -lean_inc(x_28); -lean_dec(x_21); -x_29 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_29, 0, x_28); -lean_ctor_set(x_29, 1, x_19); -x_30 = 1; -x_31 = lean_usize_add(x_4, x_30); -x_32 = lean_array_uset(x_17, x_4, x_29); -x_4 = x_31; -x_5 = x_32; -x_12 = x_27; -goto _start; +lean_object* x_78; lean_object* x_79; +x_78 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; +x_79 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_79, 0, x_78); +lean_ctor_set(x_79, 1, x_14); +x_20 = x_79; +goto block_26; } } else { -uint8_t x_34; -lean_dec(x_19); -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_2); -lean_dec(x_1); -x_34 = !lean_is_exclusive(x_20); -if (x_34 == 0) -{ -return x_20; -} -else -{ -lean_object* x_35; lean_object* x_36; lean_object* x_37; -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_alloc_ctor(1, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -return x_37; -} -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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: -{ -uint8_t x_11; -x_11 = !lean_is_exclusive(x_3); -if (x_11 == 0) -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_12 = lean_ctor_get(x_3, 0); -x_13 = lean_ctor_get(x_3, 1); -x_14 = lean_ctor_get(x_3, 2); -x_15 = lean_ctor_get(x_3, 3); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_2); -lean_inc(x_1); -x_16 = l_Lean_PersistentArray_mapMAux___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__7(x_1, x_2, x_12, x_4, x_5, 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; size_t x_19; size_t x_20; lean_object* x_21; -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_16, 1); -lean_inc(x_18); -lean_dec(x_16); -x_19 = lean_array_size(x_13); -x_20 = 0; -x_21 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__10(x_1, x_2, x_19, x_20, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_18); -if (lean_obj_tag(x_21) == 0) +lean_object* x_80; uint8_t x_81; +x_80 = lean_array_fget(x_2, x_6); +x_81 = lean_expr_eqv(x_63, x_80); +lean_dec(x_80); +lean_dec(x_63); +if (x_81 == 0) { -uint8_t x_22; -x_22 = !lean_is_exclusive(x_21); -if (x_22 == 0) +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_82 = lean_st_ref_take(x_1, x_14); +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 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_resetMaskAt(x_83, x_6); +x_86 = lean_st_ref_set(x_1, x_85, x_84); +x_87 = !lean_is_exclusive(x_86); +if (x_87 == 0) { -lean_object* x_23; -x_23 = lean_ctor_get(x_21, 0); -lean_ctor_set(x_3, 1, x_23); -lean_ctor_set(x_3, 0, x_17); -lean_ctor_set(x_21, 0, x_3); -return x_21; +lean_object* x_88; lean_object* x_89; +x_88 = lean_ctor_get(x_86, 0); +lean_dec(x_88); +x_89 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; +lean_ctor_set(x_86, 0, x_89); +x_20 = x_86; +goto block_26; } else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_21, 0); -x_25 = lean_ctor_get(x_21, 1); -lean_inc(x_25); -lean_inc(x_24); -lean_dec(x_21); -lean_ctor_set(x_3, 1, x_24); -lean_ctor_set(x_3, 0, x_17); -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_3); -lean_ctor_set(x_26, 1, x_25); -return x_26; +lean_object* x_90; lean_object* x_91; lean_object* x_92; +x_90 = lean_ctor_get(x_86, 1); +lean_inc(x_90); +lean_dec(x_86); +x_91 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; +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_20 = x_92; +goto block_26; } } else { -uint8_t x_27; -lean_dec(x_17); -lean_free_object(x_3); -lean_dec(x_15); -lean_dec(x_14); -x_27 = !lean_is_exclusive(x_21); -if (x_27 == 0) -{ -return x_21; +lean_object* x_93; lean_object* x_94; +x_93 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; +x_94 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_94, 0, x_93); +lean_ctor_set(x_94, 1, x_14); +x_20 = x_94; +goto block_26; } -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; } } } else { -uint8_t x_31; -lean_free_object(x_3); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -x_31 = !lean_is_exclusive(x_16); -if (x_31 == 0) +lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; uint8_t x_100; +lean_dec(x_27); +x_95 = lean_st_ref_take(x_1, x_14); +x_96 = lean_ctor_get(x_95, 0); +lean_inc(x_96); +x_97 = lean_ctor_get(x_95, 1); +lean_inc(x_97); +lean_dec(x_95); +x_98 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_resetMaskAt(x_96, x_6); +x_99 = lean_st_ref_set(x_1, x_98, x_97); +x_100 = !lean_is_exclusive(x_99); +if (x_100 == 0) { -return x_16; +lean_object* x_101; lean_object* x_102; +x_101 = lean_ctor_get(x_99, 0); +lean_dec(x_101); +x_102 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; +lean_ctor_set(x_99, 0, x_102); +x_20 = x_99; +goto block_26; } 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_103; lean_object* x_104; lean_object* x_105; +x_103 = lean_ctor_get(x_99, 1); +lean_inc(x_103); +lean_dec(x_99); +x_104 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___lambda__1___closed__1; +x_105 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_105, 0, x_104); +lean_ctor_set(x_105, 1, x_103); +x_20 = x_105; +goto block_26; } } -else -{ -lean_object* x_35; lean_object* x_36; lean_object* x_37; size_t x_38; lean_object* x_39; lean_object* x_40; -x_35 = lean_ctor_get(x_3, 0); -x_36 = lean_ctor_get(x_3, 1); -x_37 = lean_ctor_get(x_3, 2); -x_38 = lean_ctor_get_usize(x_3, 4); -x_39 = lean_ctor_get(x_3, 3); -lean_inc(x_39); -lean_inc(x_37); -lean_inc(x_36); -lean_inc(x_35); -lean_dec(x_3); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_2); -lean_inc(x_1); -x_40 = l_Lean_PersistentArray_mapMAux___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__7(x_1, x_2, x_35, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_40) == 0) -{ -lean_object* x_41; lean_object* x_42; size_t x_43; size_t x_44; lean_object* x_45; -x_41 = lean_ctor_get(x_40, 0); -lean_inc(x_41); -x_42 = lean_ctor_get(x_40, 1); -lean_inc(x_42); -lean_dec(x_40); -x_43 = lean_array_size(x_36); -x_44 = 0; -x_45 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__10(x_1, x_2, x_43, x_44, x_36, x_4, x_5, x_6, x_7, x_8, x_9, x_42); -if (lean_obj_tag(x_45) == 0) +block_26: { -lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_46 = lean_ctor_get(x_45, 0); -lean_inc(x_46); -x_47 = lean_ctor_get(x_45, 1); -lean_inc(x_47); -if (lean_is_exclusive(x_45)) { - lean_ctor_release(x_45, 0); - lean_ctor_release(x_45, 1); - x_48 = x_45; -} else { - lean_dec_ref(x_45); - x_48 = lean_box(0); -} -x_49 = lean_alloc_ctor(0, 4, sizeof(size_t)*1); -lean_ctor_set(x_49, 0, x_41); -lean_ctor_set(x_49, 1, x_46); -lean_ctor_set(x_49, 2, x_37); -lean_ctor_set(x_49, 3, x_39); -lean_ctor_set_usize(x_49, 4, x_38); -if (lean_is_scalar(x_48)) { - x_50 = lean_alloc_ctor(0, 2, 0); -} else { - x_50 = x_48; +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +x_23 = lean_ctor_get(x_21, 0); +lean_inc(x_23); +lean_dec(x_21); +x_24 = lean_nat_add(x_6, x_8); +lean_dec(x_6); +x_5 = x_19; +x_6 = x_24; +x_9 = x_23; +x_14 = x_22; +goto _start; } -lean_ctor_set(x_50, 0, x_49); -lean_ctor_set(x_50, 1, x_47); -return x_50; } else { -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; -lean_dec(x_41); -lean_dec(x_39); -lean_dec(x_37); -x_51 = lean_ctor_get(x_45, 0); -lean_inc(x_51); -x_52 = lean_ctor_get(x_45, 1); -lean_inc(x_52); -if (lean_is_exclusive(x_45)) { - lean_ctor_release(x_45, 0); - lean_ctor_release(x_45, 1); - x_53 = x_45; -} else { - lean_dec_ref(x_45); - x_53 = lean_box(0); -} -if (lean_is_scalar(x_53)) { - x_54 = lean_alloc_ctor(1, 2, 0); -} else { - x_54 = x_53; -} -lean_ctor_set(x_54, 0, x_51); -lean_ctor_set(x_54, 1, x_52); -return x_54; +lean_object* x_106; +lean_dec(x_6); +lean_dec(x_5); +x_106 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_106, 0, x_9); +lean_ctor_set(x_106, 1, x_14); +return x_106; } } else { -lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; -lean_dec(x_39); -lean_dec(x_37); -lean_dec(x_36); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); +lean_object* x_107; lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -x_55 = lean_ctor_get(x_40, 0); -lean_inc(x_55); -x_56 = lean_ctor_get(x_40, 1); -lean_inc(x_56); -if (lean_is_exclusive(x_40)) { - lean_ctor_release(x_40, 0); - lean_ctor_release(x_40, 1); - x_57 = x_40; -} else { - lean_dec_ref(x_40); - 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; -} +x_107 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_107, 0, x_9); +lean_ctor_set(x_107, 1, x_14); +return x_107; } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__13(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_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___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) { _start: { -uint8_t x_13; -x_13 = lean_usize_dec_lt(x_4, x_3); -if (x_13 == 0) +uint8_t x_12; +x_12 = lean_nat_dec_le(x_4, x_3); +if (x_12 == 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_object* x_13; uint8_t x_14; +x_13 = lean_unsigned_to_nat(0u); +x_14 = lean_nat_dec_eq(x_2, x_13); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_dec(x_6); +x_15 = lean_unsigned_to_nat(1u); +x_16 = lean_nat_sub(x_2, x_15); 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; -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_7); -lean_inc(x_6); -lean_inc(x_2); -lean_inc(x_1); -x_18 = l_Lean_PersistentArray_mapMAux___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__12(x_1, x_2, x_15, 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; lean_object* x_20; size_t x_21; size_t x_22; lean_object* x_23; -x_19 = lean_ctor_get(x_18, 0); +x_17 = lean_st_ref_take(x_1, 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); -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_4, x_21); -x_23 = lean_array_uset(x_17, x_4, x_19); -x_4 = x_22; -x_5 = x_23; -x_12 = x_20; +lean_dec(x_17); +x_20 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_resetMaskAt(x_18, x_3); +x_21 = lean_st_ref_set(x_1, x_20, x_19); +x_22 = lean_ctor_get(x_21, 1); +lean_inc(x_22); +lean_dec(x_21); +x_23 = lean_nat_add(x_3, x_5); +lean_dec(x_3); +x_24 = lean_box(0); +x_2 = x_16; +x_3 = x_23; +x_6 = x_24; +x_11 = x_22; goto _start; } else { -uint8_t x_25; -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_object* x_26; +lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_25 = !lean_is_exclusive(x_18); -if (x_25 == 0) -{ -return x_18; +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_6); +lean_ctor_set(x_26, 1, x_11); +return x_26; +} } 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_object* x_27; +lean_dec(x_3); +lean_dec(x_2); +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_6); +lean_ctor_set(x_27, 1, x_11); +return x_27; } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__14(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_Lean_ForEachExprWhere_visited___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { -uint8_t x_13; -x_13 = lean_usize_dec_lt(x_4, x_3); -if (x_13 == 0) +lean_object* x_8; uint8_t x_9; +x_8 = lean_st_ref_get(x_2, x_7); +x_9 = !lean_is_exclusive(x_8); +if (x_9 == 0) { -lean_object* x_14; -lean_dec(x_11); +lean_object* x_10; lean_object* x_11; size_t x_12; size_t x_13; size_t x_14; lean_object* x_15; lean_object* x_16; size_t x_17; uint8_t x_18; +x_10 = lean_ctor_get(x_8, 0); +x_11 = lean_ctor_get(x_8, 1); +x_12 = lean_ptr_addr(x_1); +x_13 = 8191; +x_14 = lean_usize_mod(x_12, x_13); +x_15 = lean_ctor_get(x_10, 0); +lean_inc(x_15); lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_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; +x_16 = lean_array_uget(x_15, x_14); +lean_dec(x_15); +x_17 = lean_ptr_addr(x_16); +lean_dec(x_16); +x_18 = lean_usize_dec_eq(x_17, x_12); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; +lean_free_object(x_8); +x_19 = lean_st_ref_take(x_2, x_11); +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_19, 1); +lean_inc(x_21); +lean_dec(x_19); +x_22 = !lean_is_exclusive(x_20); +if (x_22 == 0) +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; +x_23 = lean_ctor_get(x_20, 0); +x_24 = lean_array_uset(x_23, x_14, x_1); +lean_ctor_set(x_20, 0, x_24); +x_25 = lean_st_ref_set(x_2, x_20, x_21); +x_26 = !lean_is_exclusive(x_25); +if (x_26 == 0) +{ +lean_object* x_27; uint8_t x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_25, 0); +lean_dec(x_27); +x_28 = 0; +x_29 = lean_box(x_28); +lean_ctor_set(x_25, 0, x_29); +return x_25; } 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_array_uget(x_5, x_4); -x_16 = lean_unsigned_to_nat(0u); -x_17 = lean_array_uset(x_5, x_4, x_16); -x_18 = lean_ctor_get(x_2, 0); -lean_inc(x_18); -x_19 = l_Lean_Elab_InfoTree_substitute(x_15, x_18); -lean_inc(x_1); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -x_20 = lean_apply_7(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_20) == 0) -{ -lean_object* x_21; -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -if (lean_obj_tag(x_21) == 0) +lean_object* x_30; uint8_t x_31; lean_object* x_32; lean_object* x_33; +x_30 = lean_ctor_get(x_25, 1); +lean_inc(x_30); +lean_dec(x_25); +x_31 = 0; +x_32 = lean_box(x_31); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_30); +return x_33; +} +} +else { -lean_object* x_22; size_t x_23; size_t x_24; lean_object* x_25; -x_22 = lean_ctor_get(x_20, 1); -lean_inc(x_22); +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; lean_object* x_42; lean_object* x_43; +x_34 = lean_ctor_get(x_20, 0); +x_35 = lean_ctor_get(x_20, 1); +lean_inc(x_35); +lean_inc(x_34); lean_dec(x_20); -x_23 = 1; -x_24 = lean_usize_add(x_4, x_23); -x_25 = lean_array_uset(x_17, x_4, x_19); -x_4 = x_24; -x_5 = x_25; -x_12 = x_22; -goto _start; +x_36 = lean_array_uset(x_34, x_14, x_1); +x_37 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_37, 0, x_36); +lean_ctor_set(x_37, 1, x_35); +x_38 = lean_st_ref_set(x_2, x_37, x_21); +x_39 = lean_ctor_get(x_38, 1); +lean_inc(x_39); +if (lean_is_exclusive(x_38)) { + lean_ctor_release(x_38, 0); + lean_ctor_release(x_38, 1); + x_40 = x_38; +} else { + lean_dec_ref(x_38); + x_40 = lean_box(0); +} +x_41 = 0; +x_42 = lean_box(x_41); +if (lean_is_scalar(x_40)) { + x_43 = lean_alloc_ctor(0, 2, 0); +} else { + x_43 = x_40; +} +lean_ctor_set(x_43, 0, x_42); +lean_ctor_set(x_43, 1, x_39); +return x_43; +} } else { -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_20, 1); -lean_inc(x_27); -lean_dec(x_20); -x_28 = lean_ctor_get(x_21, 0); -lean_inc(x_28); -lean_dec(x_21); -x_29 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_29, 0, x_28); -lean_ctor_set(x_29, 1, x_19); -x_30 = 1; -x_31 = lean_usize_add(x_4, x_30); -x_32 = lean_array_uset(x_17, x_4, x_29); -x_4 = x_31; -x_5 = x_32; -x_12 = x_27; -goto _start; +uint8_t x_44; lean_object* x_45; +lean_dec(x_1); +x_44 = 1; +x_45 = lean_box(x_44); +lean_ctor_set(x_8, 0, x_45); +return x_8; } } else { -uint8_t x_34; -lean_dec(x_19); -lean_dec(x_17); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); +lean_object* x_46; lean_object* x_47; size_t x_48; size_t x_49; size_t x_50; lean_object* x_51; lean_object* x_52; size_t x_53; uint8_t x_54; +x_46 = lean_ctor_get(x_8, 0); +x_47 = lean_ctor_get(x_8, 1); +lean_inc(x_47); +lean_inc(x_46); lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_2); -lean_dec(x_1); -x_34 = !lean_is_exclusive(x_20); -if (x_34 == 0) +x_48 = lean_ptr_addr(x_1); +x_49 = 8191; +x_50 = lean_usize_mod(x_48, x_49); +x_51 = lean_ctor_get(x_46, 0); +lean_inc(x_51); +lean_dec(x_46); +x_52 = lean_array_uget(x_51, x_50); +lean_dec(x_51); +x_53 = lean_ptr_addr(x_52); +lean_dec(x_52); +x_54 = lean_usize_dec_eq(x_53, x_48); +if (x_54 == 0) { -return x_20; +lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; uint8_t x_66; lean_object* x_67; lean_object* x_68; +x_55 = lean_st_ref_take(x_2, x_47); +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); +x_59 = lean_ctor_get(x_56, 1); +lean_inc(x_59); +if (lean_is_exclusive(x_56)) { + lean_ctor_release(x_56, 0); + lean_ctor_release(x_56, 1); + x_60 = x_56; +} else { + lean_dec_ref(x_56); + x_60 = lean_box(0); +} +x_61 = lean_array_uset(x_58, x_50, x_1); +if (lean_is_scalar(x_60)) { + x_62 = lean_alloc_ctor(0, 2, 0); +} else { + x_62 = x_60; +} +lean_ctor_set(x_62, 0, x_61); +lean_ctor_set(x_62, 1, x_59); +x_63 = lean_st_ref_set(x_2, x_62, x_57); +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 = 0; +x_67 = lean_box(x_66); +if (lean_is_scalar(x_65)) { + x_68 = lean_alloc_ctor(0, 2, 0); +} else { + x_68 = x_65; +} +lean_ctor_set(x_68, 0, x_67); +lean_ctor_set(x_68, 1, x_64); +return x_68; } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; -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_alloc_ctor(1, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -return x_37; -} +uint8_t x_69; lean_object* x_70; lean_object* x_71; +lean_dec(x_1); +x_69 = 1; +x_70 = lean_box(x_69); +x_71 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_71, 0, x_70); +lean_ctor_set(x_71, 1, x_47); +return x_71; } } } } -LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapMAux___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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_ForEachExprWhere_checked___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { -if (lean_obj_tag(x_3) == 0) -{ -uint8_t x_11; -x_11 = !lean_is_exclusive(x_3); +lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_8 = lean_st_ref_get(x_2, x_7); +x_9 = lean_ctor_get(x_8, 0); +lean_inc(x_9); +x_10 = lean_ctor_get(x_9, 1); +lean_inc(x_10); +lean_dec(x_9); +x_11 = !lean_is_exclusive(x_8); if (x_11 == 0) { -lean_object* x_12; size_t x_13; size_t x_14; lean_object* x_15; -x_12 = lean_ctor_get(x_3, 0); -x_13 = lean_array_size(x_12); -x_14 = 0; -x_15 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__13(x_1, x_2, x_13, x_14, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_15) == 0) +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint64_t x_16; uint64_t x_17; uint64_t x_18; uint64_t x_19; uint64_t x_20; uint64_t x_21; uint64_t x_22; size_t x_23; size_t x_24; size_t x_25; size_t x_26; size_t x_27; lean_object* x_28; uint8_t x_29; +x_12 = lean_ctor_get(x_8, 1); +x_13 = lean_ctor_get(x_8, 0); +lean_dec(x_13); +x_14 = lean_ctor_get(x_10, 1); +lean_inc(x_14); +lean_dec(x_10); +x_15 = lean_array_get_size(x_14); +x_16 = l_Lean_Expr_hash(x_1); +x_17 = 32; +x_18 = lean_uint64_shift_right(x_16, x_17); +x_19 = lean_uint64_xor(x_16, x_18); +x_20 = 16; +x_21 = lean_uint64_shift_right(x_19, x_20); +x_22 = lean_uint64_xor(x_19, x_21); +x_23 = lean_uint64_to_usize(x_22); +x_24 = lean_usize_of_nat(x_15); +lean_dec(x_15); +x_25 = 1; +x_26 = lean_usize_sub(x_24, x_25); +x_27 = lean_usize_land(x_23, x_26); +x_28 = lean_array_uget(x_14, x_27); +lean_dec(x_14); +x_29 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_CollectLevelMVars_visitExpr___spec__1(x_1, x_28); +lean_dec(x_28); +if (x_29 == 0) { -uint8_t x_16; -x_16 = !lean_is_exclusive(x_15); -if (x_16 == 0) +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; +lean_free_object(x_8); +x_30 = lean_st_ref_take(x_2, x_12); +x_31 = lean_ctor_get(x_30, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_31, 1); +lean_inc(x_32); +x_33 = lean_ctor_get(x_30, 1); +lean_inc(x_33); +lean_dec(x_30); +x_34 = !lean_is_exclusive(x_31); +if (x_34 == 0) { -lean_object* x_17; -x_17 = lean_ctor_get(x_15, 0); -lean_ctor_set(x_3, 0, x_17); -lean_ctor_set(x_15, 0, x_3); -return x_15; +lean_object* x_35; uint8_t x_36; +x_35 = lean_ctor_get(x_31, 1); +lean_dec(x_35); +x_36 = !lean_is_exclusive(x_32); +if (x_36 == 0) +{ +lean_object* x_37; lean_object* x_38; lean_object* x_39; size_t x_40; size_t x_41; size_t x_42; lean_object* x_43; uint8_t x_44; +x_37 = lean_ctor_get(x_32, 0); +x_38 = lean_ctor_get(x_32, 1); +x_39 = lean_array_get_size(x_38); +x_40 = lean_usize_of_nat(x_39); +lean_dec(x_39); +x_41 = lean_usize_sub(x_40, x_25); +x_42 = lean_usize_land(x_23, x_41); +x_43 = lean_array_uget(x_38, x_42); +x_44 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_CollectLevelMVars_visitExpr___spec__1(x_1, x_43); +if (x_44 == 0) +{ +lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; uint8_t x_55; +x_45 = lean_unsigned_to_nat(1u); +x_46 = lean_nat_add(x_37, x_45); +lean_dec(x_37); +x_47 = lean_box(0); +x_48 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_48, 0, x_1); +lean_ctor_set(x_48, 1, x_47); +lean_ctor_set(x_48, 2, x_43); +x_49 = lean_array_uset(x_38, x_42, x_48); +x_50 = lean_unsigned_to_nat(4u); +x_51 = lean_nat_mul(x_46, x_50); +x_52 = lean_unsigned_to_nat(3u); +x_53 = lean_nat_div(x_51, x_52); +lean_dec(x_51); +x_54 = lean_array_get_size(x_49); +x_55 = lean_nat_dec_le(x_53, x_54); +lean_dec(x_54); +lean_dec(x_53); +if (x_55 == 0) +{ +lean_object* x_56; lean_object* x_57; uint8_t x_58; +x_56 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_CollectLevelMVars_visitExpr___spec__2(x_49); +lean_ctor_set(x_32, 1, x_56); +lean_ctor_set(x_32, 0, x_46); +x_57 = lean_st_ref_set(x_2, x_31, x_33); +x_58 = !lean_is_exclusive(x_57); +if (x_58 == 0) +{ +lean_object* x_59; uint8_t x_60; lean_object* x_61; +x_59 = lean_ctor_get(x_57, 0); +lean_dec(x_59); +x_60 = 0; +x_61 = lean_box(x_60); +lean_ctor_set(x_57, 0, x_61); +return x_57; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_15, 0); -x_19 = lean_ctor_get(x_15, 1); -lean_inc(x_19); -lean_inc(x_18); -lean_dec(x_15); -lean_ctor_set(x_3, 0, x_18); -x_20 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_20, 0, x_3); -lean_ctor_set(x_20, 1, x_19); -return x_20; +lean_object* x_62; uint8_t x_63; lean_object* x_64; lean_object* x_65; +x_62 = lean_ctor_get(x_57, 1); +lean_inc(x_62); +lean_dec(x_57); +x_63 = 0; +x_64 = lean_box(x_63); +x_65 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_65, 0, x_64); +lean_ctor_set(x_65, 1, x_62); +return x_65; } } else { -uint8_t x_21; -lean_free_object(x_3); -x_21 = !lean_is_exclusive(x_15); -if (x_21 == 0) +lean_object* x_66; uint8_t x_67; +lean_ctor_set(x_32, 1, x_49); +lean_ctor_set(x_32, 0, x_46); +x_66 = lean_st_ref_set(x_2, x_31, x_33); +x_67 = !lean_is_exclusive(x_66); +if (x_67 == 0) { -return x_15; +lean_object* x_68; uint8_t x_69; lean_object* x_70; +x_68 = lean_ctor_get(x_66, 0); +lean_dec(x_68); +x_69 = 0; +x_70 = lean_box(x_69); +lean_ctor_set(x_66, 0, x_70); +return x_66; } else { -lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_22 = lean_ctor_get(x_15, 0); -x_23 = lean_ctor_get(x_15, 1); -lean_inc(x_23); -lean_inc(x_22); -lean_dec(x_15); -x_24 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_24, 0, x_22); -lean_ctor_set(x_24, 1, x_23); -return x_24; +lean_object* x_71; uint8_t x_72; lean_object* x_73; lean_object* x_74; +x_71 = lean_ctor_get(x_66, 1); +lean_inc(x_71); +lean_dec(x_66); +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; } } } else { -lean_object* x_25; size_t x_26; size_t x_27; lean_object* x_28; -x_25 = lean_ctor_get(x_3, 0); -lean_inc(x_25); -lean_dec(x_3); -x_26 = lean_array_size(x_25); -x_27 = 0; -x_28 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__13(x_1, x_2, x_26, x_27, x_25, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_28) == 0) +lean_object* x_75; uint8_t x_76; +lean_dec(x_43); +lean_dec(x_1); +x_75 = lean_st_ref_set(x_2, x_31, x_33); +x_76 = !lean_is_exclusive(x_75); +if (x_76 == 0) { -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_29 = lean_ctor_get(x_28, 0); -lean_inc(x_29); -x_30 = lean_ctor_get(x_28, 1); -lean_inc(x_30); -if (lean_is_exclusive(x_28)) { - lean_ctor_release(x_28, 0); - lean_ctor_release(x_28, 1); - x_31 = x_28; -} else { - lean_dec_ref(x_28); - x_31 = lean_box(0); +lean_object* x_77; uint8_t x_78; lean_object* x_79; +x_77 = lean_ctor_get(x_75, 0); +lean_dec(x_77); +x_78 = 0; +x_79 = lean_box(x_78); +lean_ctor_set(x_75, 0, x_79); +return x_75; +} +else +{ +lean_object* x_80; uint8_t x_81; lean_object* x_82; lean_object* x_83; +x_80 = lean_ctor_get(x_75, 1); +lean_inc(x_80); +lean_dec(x_75); +x_81 = 0; +x_82 = lean_box(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_80); +return x_83; } -x_32 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_32, 0, x_29); -if (lean_is_scalar(x_31)) { - x_33 = lean_alloc_ctor(0, 2, 0); -} else { - x_33 = x_31; } -lean_ctor_set(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; -x_34 = lean_ctor_get(x_28, 0); -lean_inc(x_34); -x_35 = lean_ctor_get(x_28, 1); -lean_inc(x_35); -if (lean_is_exclusive(x_28)) { - lean_ctor_release(x_28, 0); - lean_ctor_release(x_28, 1); - x_36 = x_28; +lean_object* x_84; lean_object* x_85; lean_object* x_86; size_t x_87; size_t x_88; size_t x_89; lean_object* x_90; uint8_t x_91; +x_84 = lean_ctor_get(x_32, 0); +x_85 = lean_ctor_get(x_32, 1); +lean_inc(x_85); +lean_inc(x_84); +lean_dec(x_32); +x_86 = lean_array_get_size(x_85); +x_87 = lean_usize_of_nat(x_86); +lean_dec(x_86); +x_88 = lean_usize_sub(x_87, x_25); +x_89 = lean_usize_land(x_23, x_88); +x_90 = lean_array_uget(x_85, x_89); +x_91 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_CollectLevelMVars_visitExpr___spec__1(x_1, x_90); +if (x_91 == 0) +{ +lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; uint8_t x_102; +x_92 = lean_unsigned_to_nat(1u); +x_93 = lean_nat_add(x_84, x_92); +lean_dec(x_84); +x_94 = lean_box(0); +x_95 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_95, 0, x_1); +lean_ctor_set(x_95, 1, x_94); +lean_ctor_set(x_95, 2, x_90); +x_96 = lean_array_uset(x_85, x_89, x_95); +x_97 = lean_unsigned_to_nat(4u); +x_98 = lean_nat_mul(x_93, x_97); +x_99 = lean_unsigned_to_nat(3u); +x_100 = lean_nat_div(x_98, x_99); +lean_dec(x_98); +x_101 = lean_array_get_size(x_96); +x_102 = lean_nat_dec_le(x_100, x_101); +lean_dec(x_101); +lean_dec(x_100); +if (x_102 == 0) +{ +lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; uint8_t x_108; lean_object* x_109; lean_object* x_110; +x_103 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_CollectLevelMVars_visitExpr___spec__2(x_96); +x_104 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_104, 0, x_93); +lean_ctor_set(x_104, 1, x_103); +lean_ctor_set(x_31, 1, x_104); +x_105 = lean_st_ref_set(x_2, x_31, x_33); +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_28); - x_36 = lean_box(0); + lean_dec_ref(x_105); + x_107 = lean_box(0); } -if (lean_is_scalar(x_36)) { - x_37 = lean_alloc_ctor(1, 2, 0); +x_108 = 0; +x_109 = lean_box(x_108); +if (lean_is_scalar(x_107)) { + x_110 = lean_alloc_ctor(0, 2, 0); } else { - x_37 = x_36; -} -lean_ctor_set(x_37, 0, x_34); -lean_ctor_set(x_37, 1, x_35); -return x_37; -} + x_110 = x_107; } +lean_ctor_set(x_110, 0, x_109); +lean_ctor_set(x_110, 1, x_106); +return x_110; } else { -uint8_t x_38; -x_38 = !lean_is_exclusive(x_3); -if (x_38 == 0) -{ -lean_object* x_39; size_t x_40; size_t x_41; lean_object* x_42; -x_39 = lean_ctor_get(x_3, 0); -x_40 = lean_array_size(x_39); -x_41 = 0; -x_42 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__14(x_1, x_2, x_40, x_41, x_39, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_42) == 0) -{ -uint8_t x_43; -x_43 = !lean_is_exclusive(x_42); -if (x_43 == 0) -{ -lean_object* x_44; -x_44 = lean_ctor_get(x_42, 0); -lean_ctor_set(x_3, 0, x_44); -lean_ctor_set(x_42, 0, x_3); -return x_42; +lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; uint8_t x_115; lean_object* x_116; lean_object* x_117; +x_111 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_111, 0, x_93); +lean_ctor_set(x_111, 1, x_96); +lean_ctor_set(x_31, 1, x_111); +x_112 = lean_st_ref_set(x_2, x_31, x_33); +x_113 = lean_ctor_get(x_112, 1); +lean_inc(x_113); +if (lean_is_exclusive(x_112)) { + lean_ctor_release(x_112, 0); + lean_ctor_release(x_112, 1); + x_114 = x_112; +} else { + lean_dec_ref(x_112); + x_114 = lean_box(0); } -else -{ -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_42, 0); -x_46 = lean_ctor_get(x_42, 1); -lean_inc(x_46); -lean_inc(x_45); -lean_dec(x_42); -lean_ctor_set(x_3, 0, x_45); -x_47 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_47, 0, x_3); -lean_ctor_set(x_47, 1, x_46); -return x_47; +x_115 = 0; +x_116 = lean_box(x_115); +if (lean_is_scalar(x_114)) { + x_117 = lean_alloc_ctor(0, 2, 0); +} else { + x_117 = x_114; } +lean_ctor_set(x_117, 0, x_116); +lean_ctor_set(x_117, 1, x_113); +return x_117; } -else -{ -uint8_t x_48; -lean_free_object(x_3); -x_48 = !lean_is_exclusive(x_42); -if (x_48 == 0) -{ -return x_42; } else { -lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_49 = lean_ctor_get(x_42, 0); -x_50 = lean_ctor_get(x_42, 1); -lean_inc(x_50); -lean_inc(x_49); -lean_dec(x_42); -x_51 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_51, 0, x_49); -lean_ctor_set(x_51, 1, x_50); -return x_51; +lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; uint8_t x_122; lean_object* x_123; lean_object* x_124; +lean_dec(x_90); +lean_dec(x_1); +x_118 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_118, 0, x_84); +lean_ctor_set(x_118, 1, x_85); +lean_ctor_set(x_31, 1, x_118); +x_119 = lean_st_ref_set(x_2, x_31, x_33); +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 = 0; +x_123 = lean_box(x_122); +if (lean_is_scalar(x_121)) { + x_124 = lean_alloc_ctor(0, 2, 0); +} else { + x_124 = x_121; +} +lean_ctor_set(x_124, 0, x_123); +lean_ctor_set(x_124, 1, x_120); +return x_124; } } } else { -lean_object* x_52; size_t x_53; size_t x_54; lean_object* x_55; -x_52 = lean_ctor_get(x_3, 0); -lean_inc(x_52); -lean_dec(x_3); -x_53 = lean_array_size(x_52); -x_54 = 0; -x_55 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__14(x_1, x_2, x_53, x_54, x_52, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_55) == 0) +lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; size_t x_130; size_t x_131; size_t x_132; lean_object* x_133; uint8_t x_134; +x_125 = lean_ctor_get(x_31, 0); +lean_inc(x_125); +lean_dec(x_31); +x_126 = lean_ctor_get(x_32, 0); +lean_inc(x_126); +x_127 = lean_ctor_get(x_32, 1); +lean_inc(x_127); +if (lean_is_exclusive(x_32)) { + lean_ctor_release(x_32, 0); + lean_ctor_release(x_32, 1); + x_128 = x_32; +} else { + lean_dec_ref(x_32); + x_128 = lean_box(0); +} +x_129 = lean_array_get_size(x_127); +x_130 = lean_usize_of_nat(x_129); +lean_dec(x_129); +x_131 = lean_usize_sub(x_130, x_25); +x_132 = lean_usize_land(x_23, x_131); +x_133 = lean_array_uget(x_127, x_132); +x_134 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_CollectLevelMVars_visitExpr___spec__1(x_1, x_133); +if (x_134 == 0) { -lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_56 = lean_ctor_get(x_55, 0); -lean_inc(x_56); -x_57 = lean_ctor_get(x_55, 1); -lean_inc(x_57); -if (lean_is_exclusive(x_55)) { - lean_ctor_release(x_55, 0); - lean_ctor_release(x_55, 1); - x_58 = x_55; +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; uint8_t x_145; +x_135 = lean_unsigned_to_nat(1u); +x_136 = lean_nat_add(x_126, x_135); +lean_dec(x_126); +x_137 = lean_box(0); +x_138 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_138, 0, x_1); +lean_ctor_set(x_138, 1, x_137); +lean_ctor_set(x_138, 2, x_133); +x_139 = lean_array_uset(x_127, x_132, x_138); +x_140 = lean_unsigned_to_nat(4u); +x_141 = lean_nat_mul(x_136, x_140); +x_142 = lean_unsigned_to_nat(3u); +x_143 = lean_nat_div(x_141, x_142); +lean_dec(x_141); +x_144 = lean_array_get_size(x_139); +x_145 = lean_nat_dec_le(x_143, x_144); +lean_dec(x_144); +lean_dec(x_143); +if (x_145 == 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; uint8_t x_152; lean_object* x_153; lean_object* x_154; +x_146 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_CollectLevelMVars_visitExpr___spec__2(x_139); +if (lean_is_scalar(x_128)) { + x_147 = lean_alloc_ctor(0, 2, 0); } else { - lean_dec_ref(x_55); - x_58 = lean_box(0); + x_147 = x_128; } -x_59 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_59, 0, x_56); -if (lean_is_scalar(x_58)) { - x_60 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_147, 0, x_136); +lean_ctor_set(x_147, 1, x_146); +x_148 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_148, 0, x_125); +lean_ctor_set(x_148, 1, x_147); +x_149 = lean_st_ref_set(x_2, x_148, x_33); +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; } else { - x_60 = x_58; + lean_dec_ref(x_149); + x_151 = lean_box(0); } -lean_ctor_set(x_60, 0, x_59); -lean_ctor_set(x_60, 1, x_57); -return x_60; +x_152 = 0; +x_153 = lean_box(x_152); +if (lean_is_scalar(x_151)) { + x_154 = lean_alloc_ctor(0, 2, 0); +} else { + x_154 = x_151; +} +lean_ctor_set(x_154, 0, x_153); +lean_ctor_set(x_154, 1, x_150); +return x_154; } else { -lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; -x_61 = lean_ctor_get(x_55, 0); -lean_inc(x_61); -x_62 = lean_ctor_get(x_55, 1); -lean_inc(x_62); -if (lean_is_exclusive(x_55)) { - lean_ctor_release(x_55, 0); - lean_ctor_release(x_55, 1); - x_63 = x_55; +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_object* x_161; lean_object* x_162; +if (lean_is_scalar(x_128)) { + x_155 = lean_alloc_ctor(0, 2, 0); } else { - lean_dec_ref(x_55); - x_63 = lean_box(0); + x_155 = x_128; } -if (lean_is_scalar(x_63)) { - x_64 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_155, 0, x_136); +lean_ctor_set(x_155, 1, x_139); +x_156 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_156, 0, x_125); +lean_ctor_set(x_156, 1, x_155); +x_157 = lean_st_ref_set(x_2, x_156, x_33); +x_158 = lean_ctor_get(x_157, 1); +lean_inc(x_158); +if (lean_is_exclusive(x_157)) { + lean_ctor_release(x_157, 0); + lean_ctor_release(x_157, 1); + x_159 = x_157; } else { - x_64 = x_63; -} -lean_ctor_set(x_64, 0, x_61); -lean_ctor_set(x_64, 1, x_62); -return x_64; -} + lean_dec_ref(x_157); + x_159 = lean_box(0); } +x_160 = 0; +x_161 = lean_box(x_160); +if (lean_is_scalar(x_159)) { + x_162 = lean_alloc_ctor(0, 2, 0); +} else { + x_162 = x_159; } +lean_ctor_set(x_162, 0, x_161); +lean_ctor_set(x_162, 1, x_158); +return x_162; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__15(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) +else { -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_2); +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_dec(x_133); 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; +if (lean_is_scalar(x_128)) { + x_163 = lean_alloc_ctor(0, 2, 0); +} else { + x_163 = x_128; +} +lean_ctor_set(x_163, 0, x_126); +lean_ctor_set(x_163, 1, x_127); +x_164 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_164, 0, x_125); +lean_ctor_set(x_164, 1, x_163); +x_165 = lean_st_ref_set(x_2, x_164, x_33); +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; +} else { + lean_dec_ref(x_165); + x_167 = lean_box(0); +} +x_168 = 0; +x_169 = lean_box(x_168); +if (lean_is_scalar(x_167)) { + x_170 = lean_alloc_ctor(0, 2, 0); +} else { + x_170 = x_167; +} +lean_ctor_set(x_170, 0, x_169); +lean_ctor_set(x_170, 1, x_166); +return x_170; +} } -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_array_uget(x_5, x_4); -x_16 = lean_unsigned_to_nat(0u); -x_17 = lean_array_uset(x_5, x_4, x_16); -x_18 = lean_ctor_get(x_2, 0); -lean_inc(x_18); -x_19 = l_Lean_Elab_InfoTree_substitute(x_15, x_18); -lean_inc(x_1); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -x_20 = lean_apply_7(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_20) == 0) -{ -lean_object* x_21; -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -if (lean_obj_tag(x_21) == 0) -{ -lean_object* x_22; size_t x_23; size_t x_24; lean_object* x_25; -x_22 = lean_ctor_get(x_20, 1); -lean_inc(x_22); -lean_dec(x_20); -x_23 = 1; -x_24 = lean_usize_add(x_4, x_23); -x_25 = lean_array_uset(x_17, x_4, x_19); -x_4 = x_24; -x_5 = x_25; -x_12 = x_22; -goto _start; } else { -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_20, 1); -lean_inc(x_27); -lean_dec(x_20); -x_28 = lean_ctor_get(x_21, 0); -lean_inc(x_28); -lean_dec(x_21); -x_29 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_29, 0, x_28); -lean_ctor_set(x_29, 1, x_19); -x_30 = 1; -x_31 = lean_usize_add(x_4, x_30); -x_32 = lean_array_uset(x_17, x_4, x_29); -x_4 = x_31; -x_5 = x_32; -x_12 = x_27; -goto _start; +uint8_t x_171; lean_object* x_172; +lean_dec(x_1); +x_171 = 1; +x_172 = lean_box(x_171); +lean_ctor_set(x_8, 0, x_172); +return x_8; } } else { -uint8_t x_34; -lean_dec(x_19); -lean_dec(x_17); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); +lean_object* x_173; lean_object* x_174; lean_object* x_175; uint64_t x_176; uint64_t x_177; uint64_t x_178; uint64_t x_179; uint64_t x_180; uint64_t x_181; uint64_t x_182; size_t x_183; size_t x_184; size_t x_185; size_t x_186; size_t x_187; lean_object* x_188; uint8_t x_189; +x_173 = lean_ctor_get(x_8, 1); +lean_inc(x_173); lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_2); -lean_dec(x_1); -x_34 = !lean_is_exclusive(x_20); -if (x_34 == 0) +x_174 = lean_ctor_get(x_10, 1); +lean_inc(x_174); +lean_dec(x_10); +x_175 = lean_array_get_size(x_174); +x_176 = l_Lean_Expr_hash(x_1); +x_177 = 32; +x_178 = lean_uint64_shift_right(x_176, x_177); +x_179 = lean_uint64_xor(x_176, x_178); +x_180 = 16; +x_181 = lean_uint64_shift_right(x_179, x_180); +x_182 = lean_uint64_xor(x_179, x_181); +x_183 = lean_uint64_to_usize(x_182); +x_184 = lean_usize_of_nat(x_175); +lean_dec(x_175); +x_185 = 1; +x_186 = lean_usize_sub(x_184, x_185); +x_187 = lean_usize_land(x_183, x_186); +x_188 = lean_array_uget(x_174, x_187); +lean_dec(x_174); +x_189 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_CollectLevelMVars_visitExpr___spec__1(x_1, x_188); +lean_dec(x_188); +if (x_189 == 0) { -return x_20; +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; size_t x_200; size_t x_201; size_t x_202; lean_object* x_203; uint8_t x_204; +x_190 = lean_st_ref_take(x_2, x_173); +x_191 = lean_ctor_get(x_190, 0); +lean_inc(x_191); +x_192 = lean_ctor_get(x_191, 1); +lean_inc(x_192); +x_193 = lean_ctor_get(x_190, 1); +lean_inc(x_193); +lean_dec(x_190); +x_194 = lean_ctor_get(x_191, 0); +lean_inc(x_194); +if (lean_is_exclusive(x_191)) { + lean_ctor_release(x_191, 0); + lean_ctor_release(x_191, 1); + x_195 = x_191; +} else { + lean_dec_ref(x_191); + x_195 = lean_box(0); } -else +x_196 = lean_ctor_get(x_192, 0); +lean_inc(x_196); +x_197 = lean_ctor_get(x_192, 1); +lean_inc(x_197); +if (lean_is_exclusive(x_192)) { + lean_ctor_release(x_192, 0); + lean_ctor_release(x_192, 1); + x_198 = x_192; +} else { + lean_dec_ref(x_192); + x_198 = lean_box(0); +} +x_199 = lean_array_get_size(x_197); +x_200 = lean_usize_of_nat(x_199); +lean_dec(x_199); +x_201 = lean_usize_sub(x_200, x_185); +x_202 = lean_usize_land(x_183, x_201); +x_203 = lean_array_uget(x_197, x_202); +x_204 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_CollectLevelMVars_visitExpr___spec__1(x_1, x_203); +if (x_204 == 0) { -lean_object* x_35; lean_object* x_36; lean_object* x_37; -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_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_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; uint8_t x_215; +x_205 = lean_unsigned_to_nat(1u); +x_206 = lean_nat_add(x_196, x_205); +lean_dec(x_196); +x_207 = lean_box(0); +x_208 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_208, 0, x_1); +lean_ctor_set(x_208, 1, x_207); +lean_ctor_set(x_208, 2, x_203); +x_209 = lean_array_uset(x_197, x_202, x_208); +x_210 = lean_unsigned_to_nat(4u); +x_211 = lean_nat_mul(x_206, x_210); +x_212 = lean_unsigned_to_nat(3u); +x_213 = lean_nat_div(x_211, x_212); +lean_dec(x_211); +x_214 = lean_array_get_size(x_209); +x_215 = lean_nat_dec_le(x_213, x_214); +lean_dec(x_214); +lean_dec(x_213); +if (x_215 == 0) +{ +lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; uint8_t x_222; lean_object* x_223; lean_object* x_224; +x_216 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_CollectLevelMVars_visitExpr___spec__2(x_209); +if (lean_is_scalar(x_198)) { + x_217 = lean_alloc_ctor(0, 2, 0); +} else { + x_217 = x_198; } +lean_ctor_set(x_217, 0, x_206); +lean_ctor_set(x_217, 1, x_216); +if (lean_is_scalar(x_195)) { + x_218 = lean_alloc_ctor(0, 2, 0); +} else { + x_218 = x_195; } +lean_ctor_set(x_218, 0, x_194); +lean_ctor_set(x_218, 1, x_217); +x_219 = lean_st_ref_set(x_2, x_218, x_193); +x_220 = lean_ctor_get(x_219, 1); +lean_inc(x_220); +if (lean_is_exclusive(x_219)) { + lean_ctor_release(x_219, 0); + lean_ctor_release(x_219, 1); + x_221 = x_219; +} else { + lean_dec_ref(x_219); + x_221 = lean_box(0); } +x_222 = 0; +x_223 = lean_box(x_222); +if (lean_is_scalar(x_221)) { + x_224 = lean_alloc_ctor(0, 2, 0); +} else { + x_224 = x_221; } +lean_ctor_set(x_224, 0, x_223); +lean_ctor_set(x_224, 1, x_220); +return x_224; } -LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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: -{ -uint8_t x_11; -x_11 = !lean_is_exclusive(x_3); -if (x_11 == 0) +else { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_12 = lean_ctor_get(x_3, 0); -x_13 = lean_ctor_get(x_3, 1); -x_14 = lean_ctor_get(x_3, 2); -x_15 = lean_ctor_get(x_3, 3); -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_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; +if (lean_is_scalar(x_198)) { + x_225 = lean_alloc_ctor(0, 2, 0); +} else { + x_225 = x_198; +} +lean_ctor_set(x_225, 0, x_206); +lean_ctor_set(x_225, 1, x_209); +if (lean_is_scalar(x_195)) { + x_226 = lean_alloc_ctor(0, 2, 0); +} else { + x_226 = x_195; +} +lean_ctor_set(x_226, 0, x_194); +lean_ctor_set(x_226, 1, x_225); +x_227 = lean_st_ref_set(x_2, x_226, x_193); +x_228 = lean_ctor_get(x_227, 1); +lean_inc(x_228); +if (lean_is_exclusive(x_227)) { + lean_ctor_release(x_227, 0); + lean_ctor_release(x_227, 1); + x_229 = x_227; +} else { + lean_dec_ref(x_227); + x_229 = lean_box(0); +} +x_230 = 0; +x_231 = lean_box(x_230); +if (lean_is_scalar(x_229)) { + x_232 = lean_alloc_ctor(0, 2, 0); +} else { + x_232 = x_229; +} +lean_ctor_set(x_232, 0, x_231); +lean_ctor_set(x_232, 1, x_228); +return x_232; +} +} +else +{ +lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; uint8_t x_238; lean_object* x_239; lean_object* x_240; +lean_dec(x_203); +lean_dec(x_1); +if (lean_is_scalar(x_198)) { + x_233 = lean_alloc_ctor(0, 2, 0); +} else { + x_233 = x_198; +} +lean_ctor_set(x_233, 0, x_196); +lean_ctor_set(x_233, 1, x_197); +if (lean_is_scalar(x_195)) { + x_234 = lean_alloc_ctor(0, 2, 0); +} else { + x_234 = x_195; +} +lean_ctor_set(x_234, 0, x_194); +lean_ctor_set(x_234, 1, x_233); +x_235 = lean_st_ref_set(x_2, x_234, x_193); +x_236 = lean_ctor_get(x_235, 1); +lean_inc(x_236); +if (lean_is_exclusive(x_235)) { + lean_ctor_release(x_235, 0); + lean_ctor_release(x_235, 1); + x_237 = x_235; +} else { + lean_dec_ref(x_235); + x_237 = lean_box(0); +} +x_238 = 0; +x_239 = lean_box(x_238); +if (lean_is_scalar(x_237)) { + x_240 = lean_alloc_ctor(0, 2, 0); +} else { + x_240 = x_237; +} +lean_ctor_set(x_240, 0, x_239); +lean_ctor_set(x_240, 1, x_236); +return x_240; +} +} +else +{ +uint8_t x_241; lean_object* x_242; lean_object* x_243; +lean_dec(x_1); +x_241 = 1; +x_242 = lean_box(x_241); +x_243 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_243, 0, x_242); +lean_ctor_set(x_243, 1, x_173); +return x_243; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +switch (lean_obj_tag(x_1)) { +case 5: +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_1, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_1, 1); +lean_inc(x_13); +lean_dec(x_1); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_3); lean_inc(x_2); -lean_inc(x_1); -x_16 = l_Lean_PersistentArray_mapMAux___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__12(x_1, x_2, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_16) == 0) +x_14 = l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6(x_2, x_3, x_4, x_12, x_6, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_14) == 0) { -lean_object* x_17; lean_object* x_18; size_t x_19; size_t x_20; lean_object* x_21; -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_16, 1); -lean_inc(x_18); -lean_dec(x_16); -x_19 = lean_array_size(x_13); -x_20 = 0; -x_21 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__15(x_1, x_2, x_19, x_20, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_18); -if (lean_obj_tag(x_21) == 0) +lean_object* x_15; lean_object* x_16; +x_15 = lean_ctor_get(x_14, 1); +lean_inc(x_15); +lean_dec(x_14); +x_16 = l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6(x_2, x_3, x_4, x_13, x_6, x_7, x_8, x_9, x_10, x_15); +return x_16; +} +else { -uint8_t x_22; -x_22 = !lean_is_exclusive(x_21); -if (x_22 == 0) +uint8_t x_17; +lean_dec(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +x_17 = !lean_is_exclusive(x_14); +if (x_17 == 0) { -lean_object* x_23; -x_23 = lean_ctor_get(x_21, 0); -lean_ctor_set(x_3, 1, x_23); -lean_ctor_set(x_3, 0, x_17); -lean_ctor_set(x_21, 0, x_3); -return x_21; +return x_14; } else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_21, 0); -x_25 = lean_ctor_get(x_21, 1); -lean_inc(x_25); -lean_inc(x_24); -lean_dec(x_21); -lean_ctor_set(x_3, 1, x_24); -lean_ctor_set(x_3, 0, x_17); -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_3); -lean_ctor_set(x_26, 1, x_25); -return x_26; +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_14, 0); +x_19 = lean_ctor_get(x_14, 1); +lean_inc(x_19); +lean_inc(x_18); +lean_dec(x_14); +x_20 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_20, 0, x_18); +lean_ctor_set(x_20, 1, x_19); +return x_20; +} +} } +case 6: +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +x_22 = lean_ctor_get(x_1, 2); +lean_inc(x_22); +lean_dec(x_1); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_3); +lean_inc(x_2); +x_23 = l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6(x_2, x_3, x_4, x_21, x_6, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_23) == 0) +{ +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_23, 1); +lean_inc(x_24); +lean_dec(x_23); +x_25 = l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6(x_2, x_3, x_4, x_22, x_6, x_7, x_8, x_9, x_10, x_24); +return x_25; } else { -uint8_t x_27; -lean_dec(x_17); -lean_free_object(x_3); -lean_dec(x_15); -lean_dec(x_14); -x_27 = !lean_is_exclusive(x_21); -if (x_27 == 0) +uint8_t x_26; +lean_dec(x_22); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +x_26 = !lean_is_exclusive(x_23); +if (x_26 == 0) { -return x_21; +return x_23; } 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_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_23, 0); +x_28 = lean_ctor_get(x_23, 1); 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_inc(x_27); +lean_dec(x_23); +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; } } } +case 7: +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_1, 1); +lean_inc(x_30); +x_31 = lean_ctor_get(x_1, 2); +lean_inc(x_31); +lean_dec(x_1); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_3); +lean_inc(x_2); +x_32 = l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6(x_2, x_3, x_4, x_30, x_6, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_32) == 0) +{ +lean_object* x_33; lean_object* x_34; +x_33 = lean_ctor_get(x_32, 1); +lean_inc(x_33); +lean_dec(x_32); +x_34 = l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6(x_2, x_3, x_4, x_31, x_6, x_7, x_8, x_9, x_10, x_33); +return x_34; +} else { -uint8_t x_31; -lean_free_object(x_3); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); +uint8_t x_35; +lean_dec(x_31); +lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_31 = !lean_is_exclusive(x_16); -if (x_31 == 0) +x_35 = !lean_is_exclusive(x_32); +if (x_35 == 0) { -return x_16; +return x_32; } 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_36; lean_object* x_37; lean_object* x_38; +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_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 +case 8: { -lean_object* x_35; lean_object* x_36; lean_object* x_37; size_t x_38; lean_object* x_39; lean_object* x_40; -x_35 = lean_ctor_get(x_3, 0); -x_36 = lean_ctor_get(x_3, 1); -x_37 = lean_ctor_get(x_3, 2); -x_38 = lean_ctor_get_usize(x_3, 4); -x_39 = lean_ctor_get(x_3, 3); +lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_39 = lean_ctor_get(x_1, 1); lean_inc(x_39); -lean_inc(x_37); -lean_inc(x_36); -lean_inc(x_35); -lean_dec(x_3); +x_40 = lean_ctor_get(x_1, 2); +lean_inc(x_40); +x_41 = lean_ctor_get(x_1, 3); +lean_inc(x_41); +lean_dec(x_1); +lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); +lean_inc(x_3); lean_inc(x_2); -lean_inc(x_1); -x_40 = l_Lean_PersistentArray_mapMAux___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__12(x_1, x_2, x_35, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_40) == 0) +x_42 = l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6(x_2, x_3, x_4, x_39, x_6, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_42) == 0) { -lean_object* x_41; lean_object* x_42; size_t x_43; size_t x_44; lean_object* x_45; -x_41 = lean_ctor_get(x_40, 0); -lean_inc(x_41); -x_42 = lean_ctor_get(x_40, 1); -lean_inc(x_42); -lean_dec(x_40); -x_43 = lean_array_size(x_36); -x_44 = 0; -x_45 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__15(x_1, x_2, x_43, x_44, x_36, x_4, x_5, x_6, x_7, x_8, x_9, x_42); -if (lean_obj_tag(x_45) == 0) +lean_object* x_43; lean_object* x_44; +x_43 = lean_ctor_get(x_42, 1); +lean_inc(x_43); +lean_dec(x_42); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_3); +lean_inc(x_2); +x_44 = l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6(x_2, x_3, x_4, x_40, x_6, x_7, x_8, x_9, x_10, x_43); +if (lean_obj_tag(x_44) == 0) { -lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_46 = lean_ctor_get(x_45, 0); -lean_inc(x_46); -x_47 = lean_ctor_get(x_45, 1); -lean_inc(x_47); -if (lean_is_exclusive(x_45)) { - lean_ctor_release(x_45, 0); - lean_ctor_release(x_45, 1); - x_48 = x_45; -} else { - lean_dec_ref(x_45); - x_48 = lean_box(0); +lean_object* x_45; lean_object* x_46; +x_45 = lean_ctor_get(x_44, 1); +lean_inc(x_45); +lean_dec(x_44); +x_46 = l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6(x_2, x_3, x_4, x_41, x_6, x_7, x_8, x_9, x_10, x_45); +return x_46; } -x_49 = lean_alloc_ctor(0, 4, sizeof(size_t)*1); -lean_ctor_set(x_49, 0, x_41); -lean_ctor_set(x_49, 1, x_46); -lean_ctor_set(x_49, 2, x_37); -lean_ctor_set(x_49, 3, x_39); -lean_ctor_set_usize(x_49, 4, x_38); -if (lean_is_scalar(x_48)) { - x_50 = lean_alloc_ctor(0, 2, 0); -} else { - x_50 = x_48; +else +{ +uint8_t x_47; +lean_dec(x_41); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +x_47 = !lean_is_exclusive(x_44); +if (x_47 == 0) +{ +return x_44; } -lean_ctor_set(x_50, 0, x_49); -lean_ctor_set(x_50, 1, x_47); +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; } +} +} else { -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +uint8_t x_51; lean_dec(x_41); -lean_dec(x_39); -lean_dec(x_37); -x_51 = lean_ctor_get(x_45, 0); -lean_inc(x_51); -x_52 = lean_ctor_get(x_45, 1); +lean_dec(x_40); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +x_51 = !lean_is_exclusive(x_42); +if (x_51 == 0) +{ +return x_42; +} +else +{ +lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_52 = lean_ctor_get(x_42, 0); +x_53 = lean_ctor_get(x_42, 1); +lean_inc(x_53); lean_inc(x_52); -if (lean_is_exclusive(x_45)) { - lean_ctor_release(x_45, 0); - lean_ctor_release(x_45, 1); - x_53 = x_45; -} else { - lean_dec_ref(x_45); - x_53 = lean_box(0); +lean_dec(x_42); +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; } -if (lean_is_scalar(x_53)) { - x_54 = lean_alloc_ctor(1, 2, 0); -} else { - x_54 = x_53; } -lean_ctor_set(x_54, 0, x_51); -lean_ctor_set(x_54, 1, x_52); -return x_54; } +case 10: +{ +lean_object* x_55; lean_object* x_56; +x_55 = lean_ctor_get(x_1, 1); +lean_inc(x_55); +lean_dec(x_1); +x_56 = l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6(x_2, x_3, x_4, x_55, x_6, x_7, x_8, x_9, x_10, x_11); +return x_56; } -else +case 11: { -lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; -lean_dec(x_39); -lean_dec(x_37); -lean_dec(x_36); +lean_object* x_57; lean_object* x_58; +x_57 = lean_ctor_get(x_1, 2); +lean_inc(x_57); +lean_dec(x_1); +x_58 = l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6(x_2, x_3, x_4, x_57, x_6, x_7, x_8, x_9, x_10, x_11); +return x_58; +} +default: +{ +lean_object* x_59; lean_object* x_60; +lean_dec(x_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_55 = lean_ctor_get(x_40, 0); -lean_inc(x_55); -x_56 = lean_ctor_get(x_40, 1); -lean_inc(x_56); -if (lean_is_exclusive(x_40)) { - lean_ctor_release(x_40, 0); - lean_ctor_release(x_40, 1); - x_57 = x_40; -} else { - lean_dec_ref(x_40); - 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; +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_11); +return x_60; } } } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__5___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_11 = l_Lean_Elab_getResetInfoTrees___at_Lean_Elab_Term_withDeclName___spec__3___rarg(x_9, x_10); +lean_object* x_11; lean_object* x_12; uint8_t x_13; +lean_inc(x_4); +x_11 = l_Lean_ForEachExprWhere_visited___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__7(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); +x_13 = lean_unbox(x_12); +lean_dec(x_12); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_14 = lean_ctor_get(x_11, 1); +lean_inc(x_14); lean_dec(x_11); +lean_inc(x_1); +lean_inc(x_4); +x_15 = lean_apply_1(x_1, x_4); +x_16 = lean_unbox(x_15); +lean_dec(x_15); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; +x_17 = lean_box(0); +x_18 = l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6___lambda__1(x_4, x_1, x_2, x_3, x_17, x_5, x_6, x_7, x_8, x_9, x_14); +return x_18; +} +else +{ +lean_object* x_19; lean_object* x_20; uint8_t x_21; +lean_inc(x_4); +x_19 = l_Lean_ForEachExprWhere_checked___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__8(x_4, x_5, x_6, x_7, x_8, x_9, x_14); +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +x_21 = lean_unbox(x_20); +lean_dec(x_20); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; +x_22 = lean_ctor_get(x_19, 1); +lean_inc(x_22); +lean_dec(x_19); +lean_inc(x_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); -x_14 = lean_apply_7(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_13); -if (lean_obj_tag(x_14) == 0) +x_23 = lean_apply_6(x_2, x_4, x_6, x_7, x_8, x_9, x_22); +if (lean_obj_tag(x_23) == 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; -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_9, x_16); -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_17, 1); -lean_inc(x_19); -lean_dec(x_17); -x_20 = lean_ctor_get(x_18, 6); -lean_inc(x_20); -lean_dec(x_18); -x_21 = lean_ctor_get(x_20, 1); -lean_inc(x_21); -lean_inc(x_9); -x_22 = l_Lean_PersistentArray_mapM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__6(x_2, x_20, x_21, x_4, x_5, x_6, x_7, x_8, x_9, x_19); -if (lean_obj_tag(x_22) == 0) +if (x_3 == 0) { -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -x_24 = lean_ctor_get(x_22, 1); +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_23, 1); lean_inc(x_24); -lean_dec(x_22); -x_25 = lean_st_ref_take(x_9, x_24); -x_26 = lean_ctor_get(x_25, 0); -lean_inc(x_26); -x_27 = lean_ctor_get(x_26, 6); -lean_inc(x_27); -x_28 = lean_ctor_get(x_25, 1); -lean_inc(x_28); -lean_dec(x_25); -x_29 = !lean_is_exclusive(x_26); -if (x_29 == 0) -{ -lean_object* x_30; uint8_t x_31; -x_30 = lean_ctor_get(x_26, 6); -lean_dec(x_30); -x_31 = !lean_is_exclusive(x_27); -if (x_31 == 0) -{ -lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; -x_32 = lean_ctor_get(x_27, 1); -lean_dec(x_32); -x_33 = l_Lean_PersistentArray_append___rarg(x_12, x_23); lean_dec(x_23); -lean_ctor_set(x_27, 1, x_33); -x_34 = lean_st_ref_set(x_9, x_26, x_28); -lean_dec(x_9); -x_35 = !lean_is_exclusive(x_34); -if (x_35 == 0) -{ -lean_object* x_36; -x_36 = lean_ctor_get(x_34, 0); -lean_dec(x_36); -lean_ctor_set(x_34, 0, x_15); -return x_34; +x_25 = lean_box(0); +x_26 = l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6___lambda__1(x_4, x_1, x_2, x_3, x_25, x_5, x_6, x_7, x_8, x_9, x_24); +return x_26; } else { -lean_object* x_37; lean_object* x_38; -x_37 = lean_ctor_get(x_34, 1); -lean_inc(x_37); -lean_dec(x_34); -x_38 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_38, 0, x_15); -lean_ctor_set(x_38, 1, x_37); -return x_38; -} +uint8_t x_27; +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_27 = !lean_is_exclusive(x_23); +if (x_27 == 0) +{ +lean_object* x_28; lean_object* x_29; +x_28 = lean_ctor_get(x_23, 0); +lean_dec(x_28); +x_29 = lean_box(0); +lean_ctor_set(x_23, 0, x_29); +return x_23; } else { -uint8_t x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_39 = lean_ctor_get_uint8(x_27, sizeof(void*)*2); -x_40 = lean_ctor_get(x_27, 0); -lean_inc(x_40); -lean_dec(x_27); -x_41 = l_Lean_PersistentArray_append___rarg(x_12, x_23); +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_23, 1); +lean_inc(x_30); lean_dec(x_23); -x_42 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_42, 0, x_40); -lean_ctor_set(x_42, 1, x_41); -lean_ctor_set_uint8(x_42, sizeof(void*)*2, x_39); -lean_ctor_set(x_26, 6, x_42); -x_43 = lean_st_ref_set(x_9, x_26, x_28); -lean_dec(x_9); -x_44 = lean_ctor_get(x_43, 1); -lean_inc(x_44); -if (lean_is_exclusive(x_43)) { - lean_ctor_release(x_43, 0); - lean_ctor_release(x_43, 1); - x_45 = x_43; -} else { - lean_dec_ref(x_43); - x_45 = lean_box(0); -} -if (lean_is_scalar(x_45)) { - x_46 = lean_alloc_ctor(0, 2, 0); -} else { - x_46 = x_45; +x_31 = lean_box(0); +x_32 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_32, 0, x_31); +lean_ctor_set(x_32, 1, x_30); +return x_32; } -lean_ctor_set(x_46, 0, x_15); -lean_ctor_set(x_46, 1, x_44); -return x_46; } } else { -lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; uint8_t x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_47 = lean_ctor_get(x_26, 0); -x_48 = lean_ctor_get(x_26, 1); -x_49 = lean_ctor_get(x_26, 2); -x_50 = lean_ctor_get(x_26, 3); -x_51 = lean_ctor_get(x_26, 4); -x_52 = lean_ctor_get(x_26, 5); -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_dec(x_26); -x_53 = lean_ctor_get_uint8(x_27, sizeof(void*)*2); -x_54 = lean_ctor_get(x_27, 0); -lean_inc(x_54); -if (lean_is_exclusive(x_27)) { - lean_ctor_release(x_27, 0); - lean_ctor_release(x_27, 1); - x_55 = x_27; -} else { - lean_dec_ref(x_27); - x_55 = lean_box(0); +uint8_t x_33; +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_33 = !lean_is_exclusive(x_23); +if (x_33 == 0) +{ +return x_23; } -x_56 = l_Lean_PersistentArray_append___rarg(x_12, x_23); +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_23, 0); +x_35 = lean_ctor_get(x_23, 1); +lean_inc(x_35); +lean_inc(x_34); lean_dec(x_23); -if (lean_is_scalar(x_55)) { - x_57 = lean_alloc_ctor(0, 2, 1); -} else { - x_57 = x_55; +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_ctor_set(x_57, 0, x_54); -lean_ctor_set(x_57, 1, x_56); -lean_ctor_set_uint8(x_57, sizeof(void*)*2, x_53); -x_58 = lean_alloc_ctor(0, 7, 0); -lean_ctor_set(x_58, 0, x_47); -lean_ctor_set(x_58, 1, x_48); -lean_ctor_set(x_58, 2, x_49); -lean_ctor_set(x_58, 3, x_50); -lean_ctor_set(x_58, 4, x_51); -lean_ctor_set(x_58, 5, x_52); -lean_ctor_set(x_58, 6, x_57); -x_59 = lean_st_ref_set(x_9, x_58, x_28); -lean_dec(x_9); -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; -} else { - lean_dec_ref(x_59); - x_61 = lean_box(0); } -if (lean_is_scalar(x_61)) { - x_62 = lean_alloc_ctor(0, 2, 0); -} else { - x_62 = x_61; } -lean_ctor_set(x_62, 0, x_15); -lean_ctor_set(x_62, 1, x_60); -return x_62; +else +{ +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_19, 1); +lean_inc(x_37); +lean_dec(x_19); +x_38 = lean_box(0); +x_39 = l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6___lambda__1(x_4, x_1, x_2, x_3, x_38, x_5, x_6, x_7, x_8, x_9, x_37); +return x_39; +} } } else { -uint8_t x_63; -lean_dec(x_15); -lean_dec(x_12); +uint8_t x_40; lean_dec(x_9); -x_63 = !lean_is_exclusive(x_22); -if (x_63 == 0) +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_40 = !lean_is_exclusive(x_11); +if (x_40 == 0) { -return x_22; +lean_object* x_41; lean_object* x_42; +x_41 = lean_ctor_get(x_11, 0); +lean_dec(x_41); +x_42 = lean_box(0); +lean_ctor_set(x_11, 0, x_42); +return x_11; } else { -lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_64 = lean_ctor_get(x_22, 0); -x_65 = lean_ctor_get(x_22, 1); -lean_inc(x_65); -lean_inc(x_64); -lean_dec(x_22); -x_66 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_66, 0, x_64); -lean_ctor_set(x_66, 1, x_65); -return x_66; +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_11, 1); +lean_inc(x_43); +lean_dec(x_11); +x_44 = lean_box(0); +x_45 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_45, 0, x_44); +lean_ctor_set(x_45, 1, x_43); +return x_45; } } } -else +} +LEAN_EXPORT lean_object* l_Lean_ForEachExprWhere_visit___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: { -lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; -x_67 = lean_ctor_get(x_14, 0); -lean_inc(x_67); -x_68 = lean_ctor_get(x_14, 1); -lean_inc(x_68); +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = l_Lean_ForEachExprWhere_initCache; +x_11 = lean_st_mk_ref(x_10, 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 = l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6(x_1, x_2, x_4, x_3, x_12, x_5, x_6, x_7, x_8, x_13); +if (lean_obj_tag(x_14) == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); lean_dec(x_14); -x_69 = lean_st_ref_get(x_9, x_68); -x_70 = lean_ctor_get(x_69, 0); -lean_inc(x_70); -x_71 = lean_ctor_get(x_69, 1); -lean_inc(x_71); -lean_dec(x_69); -x_72 = lean_ctor_get(x_70, 6); -lean_inc(x_72); -lean_dec(x_70); -x_73 = lean_ctor_get(x_72, 1); -lean_inc(x_73); -lean_inc(x_9); -x_74 = l_Lean_PersistentArray_mapM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__11(x_2, x_72, x_73, x_4, x_5, x_6, x_7, x_8, x_9, x_71); -if (lean_obj_tag(x_74) == 0) +x_17 = lean_st_ref_get(x_12, x_16); +lean_dec(x_12); +x_18 = !lean_is_exclusive(x_17); +if (x_18 == 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; uint8_t x_81; -x_75 = lean_ctor_get(x_74, 0); -lean_inc(x_75); -x_76 = lean_ctor_get(x_74, 1); -lean_inc(x_76); -lean_dec(x_74); -x_77 = lean_st_ref_take(x_9, x_76); -x_78 = lean_ctor_get(x_77, 0); -lean_inc(x_78); -x_79 = lean_ctor_get(x_78, 6); -lean_inc(x_79); -x_80 = lean_ctor_get(x_77, 1); -lean_inc(x_80); -lean_dec(x_77); -x_81 = !lean_is_exclusive(x_78); -if (x_81 == 0) +lean_object* x_19; +x_19 = lean_ctor_get(x_17, 0); +lean_dec(x_19); +lean_ctor_set(x_17, 0, x_15); +return x_17; +} +else { -lean_object* x_82; uint8_t x_83; -x_82 = lean_ctor_get(x_78, 6); -lean_dec(x_82); -x_83 = !lean_is_exclusive(x_79); -if (x_83 == 0) +lean_object* x_20; lean_object* x_21; +x_20 = lean_ctor_get(x_17, 1); +lean_inc(x_20); +lean_dec(x_17); +x_21 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_21, 0, x_15); +lean_ctor_set(x_21, 1, x_20); +return x_21; +} +} +else { -lean_object* x_84; lean_object* x_85; lean_object* x_86; uint8_t x_87; -x_84 = lean_ctor_get(x_79, 1); -lean_dec(x_84); -x_85 = l_Lean_PersistentArray_append___rarg(x_12, x_75); -lean_dec(x_75); -lean_ctor_set(x_79, 1, x_85); -x_86 = lean_st_ref_set(x_9, x_78, x_80); -lean_dec(x_9); -x_87 = !lean_is_exclusive(x_86); -if (x_87 == 0) +uint8_t x_22; +lean_dec(x_12); +x_22 = !lean_is_exclusive(x_14); +if (x_22 == 0) { -lean_object* x_88; -x_88 = lean_ctor_get(x_86, 0); -lean_dec(x_88); -lean_ctor_set_tag(x_86, 1); -lean_ctor_set(x_86, 0, x_67); -return x_86; +return x_14; } else { -lean_object* x_89; lean_object* x_90; -x_89 = lean_ctor_get(x_86, 1); -lean_inc(x_89); -lean_dec(x_86); -x_90 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_90, 0, x_67); -lean_ctor_set(x_90, 1, x_89); -return x_90; +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_14, 0); +x_24 = lean_ctor_get(x_14, 1); +lean_inc(x_24); +lean_inc(x_23); +lean_dec(x_14); +x_25 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +return x_25; +} +} +} } +LEAN_EXPORT uint8_t l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__9___lambda__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; uint8_t x_5; +x_3 = lean_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_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_91 = lean_ctor_get_uint8(x_79, sizeof(void*)*2); -x_92 = lean_ctor_get(x_79, 0); -lean_inc(x_92); -lean_dec(x_79); -x_93 = l_Lean_PersistentArray_append___rarg(x_12, x_75); -lean_dec(x_75); -x_94 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_94, 0, x_92); -lean_ctor_set(x_94, 1, x_93); -lean_ctor_set_uint8(x_94, sizeof(void*)*2, x_91); -lean_ctor_set(x_78, 6, x_94); -x_95 = lean_st_ref_set(x_9, x_78, x_80); -lean_dec(x_9); -x_96 = lean_ctor_get(x_95, 1); -lean_inc(x_96); -if (lean_is_exclusive(x_95)) { - lean_ctor_release(x_95, 0); - lean_ctor_release(x_95, 1); - x_97 = x_95; -} else { - lean_dec_ref(x_95); - x_97 = lean_box(0); +size_t x_7; size_t x_8; uint8_t x_9; +x_7 = 0; +x_8 = lean_usize_of_nat(x_3); +lean_dec(x_3); +x_9 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__2(x_2, x_1, x_7, x_8); +return x_9; } -if (lean_is_scalar(x_97)) { - x_98 = lean_alloc_ctor(1, 2, 0); -} else { - x_98 = x_97; - lean_ctor_set_tag(x_98, 1); } -lean_ctor_set(x_98, 0, x_67); -lean_ctor_set(x_98, 1, x_96); -return x_98; } +LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__9___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_12 = lean_unsigned_to_nat(0u); +x_13 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_6, x_12); +lean_inc(x_13); +x_14 = lean_mk_array(x_13, x_1); +x_15 = lean_unsigned_to_nat(1u); +x_16 = lean_nat_sub(x_13, x_15); +lean_dec(x_13); +x_17 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_6, x_14, x_16); +x_18 = lean_array_get_size(x_17); +x_19 = lean_box(0); +lean_inc(x_18); +x_20 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__3(x_2, x_3, x_17, x_18, x_18, x_4, x_18, x_15, x_19, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_17); +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +lean_inc(x_5); +x_22 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__4(x_2, x_5, x_18, x_5, x_15, x_19, x_7, x_8, x_9, x_10, x_21); +lean_dec(x_5); +x_23 = !lean_is_exclusive(x_22); +if (x_23 == 0) +{ +lean_object* x_24; +x_24 = lean_ctor_get(x_22, 0); +lean_dec(x_24); +lean_ctor_set(x_22, 0, x_19); +return x_22; } 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; 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; lean_object* x_113; lean_object* x_114; -x_99 = lean_ctor_get(x_78, 0); -x_100 = lean_ctor_get(x_78, 1); -x_101 = lean_ctor_get(x_78, 2); -x_102 = lean_ctor_get(x_78, 3); -x_103 = lean_ctor_get(x_78, 4); -x_104 = lean_ctor_get(x_78, 5); -lean_inc(x_104); -lean_inc(x_103); -lean_inc(x_102); -lean_inc(x_101); -lean_inc(x_100); -lean_inc(x_99); -lean_dec(x_78); -x_105 = lean_ctor_get_uint8(x_79, sizeof(void*)*2); -x_106 = lean_ctor_get(x_79, 0); -lean_inc(x_106); -if (lean_is_exclusive(x_79)) { - lean_ctor_release(x_79, 0); - lean_ctor_release(x_79, 1); - x_107 = x_79; -} else { - lean_dec_ref(x_79); - x_107 = lean_box(0); -} -x_108 = l_Lean_PersistentArray_append___rarg(x_12, x_75); -lean_dec(x_75); -if (lean_is_scalar(x_107)) { - x_109 = lean_alloc_ctor(0, 2, 1); -} else { - x_109 = x_107; +lean_object* x_25; lean_object* x_26; +x_25 = lean_ctor_get(x_22, 1); +lean_inc(x_25); +lean_dec(x_22); +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_19); +lean_ctor_set(x_26, 1, x_25); +return x_26; } -lean_ctor_set(x_109, 0, x_106); -lean_ctor_set(x_109, 1, x_108); -lean_ctor_set_uint8(x_109, sizeof(void*)*2, x_105); -x_110 = lean_alloc_ctor(0, 7, 0); -lean_ctor_set(x_110, 0, x_99); -lean_ctor_set(x_110, 1, x_100); -lean_ctor_set(x_110, 2, x_101); -lean_ctor_set(x_110, 3, x_102); -lean_ctor_set(x_110, 4, x_103); -lean_ctor_set(x_110, 5, x_104); -lean_ctor_set(x_110, 6, x_109); -x_111 = lean_st_ref_set(x_9, x_110, x_80); -lean_dec(x_9); -x_112 = lean_ctor_get(x_111, 1); -lean_inc(x_112); -if (lean_is_exclusive(x_111)) { - lean_ctor_release(x_111, 0); - lean_ctor_release(x_111, 1); - x_113 = x_111; -} else { - lean_dec_ref(x_111); - x_113 = lean_box(0); } -if (lean_is_scalar(x_113)) { - x_114 = lean_alloc_ctor(1, 2, 0); -} else { - x_114 = x_113; - lean_ctor_set_tag(x_114, 1); } -lean_ctor_set(x_114, 0, x_67); -lean_ctor_set(x_114, 1, x_112); -return x_114; +LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, size_t x_8, size_t x_9, lean_object* x_10, 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); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_10); +lean_ctor_set(x_17, 1, x_15); +return x_17; } +else +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; +lean_dec(x_10); +x_18 = lean_ctor_get(x_7, 0); +x_19 = lean_array_uget(x_18, x_9); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +x_20 = lean_infer_type(x_19, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_20) == 0) +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; lean_object* x_26; +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +lean_inc(x_2); +x_23 = lean_alloc_closure((void*)(l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__9___lambda__1___boxed), 2, 1); +lean_closure_set(x_23, 0, x_2); +lean_inc(x_3); +lean_inc(x_1); +lean_inc(x_6); +lean_inc(x_4); +lean_inc(x_5); +x_24 = lean_alloc_closure((void*)(l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__9___lambda__2___boxed), 11, 5); +lean_closure_set(x_24, 0, x_5); +lean_closure_set(x_24, 1, x_4); +lean_closure_set(x_24, 2, x_6); +lean_closure_set(x_24, 3, x_1); +lean_closure_set(x_24, 4, x_3); +x_25 = 1; +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +x_26 = l_Lean_ForEachExprWhere_visit___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__5(x_23, x_24, x_21, x_25, x_11, x_12, x_13, x_14, x_22); +if (lean_obj_tag(x_26) == 0) +{ +lean_object* x_27; size_t x_28; size_t x_29; lean_object* x_30; +x_27 = lean_ctor_get(x_26, 1); +lean_inc(x_27); +lean_dec(x_26); +x_28 = 1; +x_29 = lean_usize_add(x_9, x_28); +x_30 = lean_box(0); +x_9 = x_29; +x_10 = x_30; +x_15 = x_27; +goto _start; } else { -uint8_t x_115; -lean_dec(x_67); +uint8_t x_32; +lean_dec(x_14); +lean_dec(x_13); lean_dec(x_12); -lean_dec(x_9); -x_115 = !lean_is_exclusive(x_74); -if (x_115 == 0) +lean_dec(x_11); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_32 = !lean_is_exclusive(x_26); +if (x_32 == 0) { -return x_74; +return x_26; } else { -lean_object* x_116; lean_object* x_117; lean_object* x_118; -x_116 = lean_ctor_get(x_74, 0); -x_117 = lean_ctor_get(x_74, 1); -lean_inc(x_117); -lean_inc(x_116); -lean_dec(x_74); -x_118 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_118, 0, x_116); -lean_ctor_set(x_118, 1, x_117); -return x_118; -} -} +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_26, 0); +x_34 = lean_ctor_get(x_26, 1); +lean_inc(x_34); +lean_inc(x_33); +lean_dec(x_26); +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +return x_35; } } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_10 = lean_st_ref_get(x_8, x_9); -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -x_12 = lean_ctor_get(x_11, 6); -lean_inc(x_12); -lean_dec(x_11); -x_13 = lean_ctor_get_uint8(x_12, sizeof(void*)*2); +uint8_t x_36; +lean_dec(x_14); +lean_dec(x_13); lean_dec(x_12); -if (x_13 == 0) -{ -lean_object* x_14; lean_object* x_15; +lean_dec(x_11); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); -x_14 = lean_ctor_get(x_10, 1); -lean_inc(x_14); -lean_dec(x_10); -x_15 = lean_apply_7(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_14); -if (lean_obj_tag(x_15) == 0) -{ -uint8_t x_16; -x_16 = !lean_is_exclusive(x_15); -if (x_16 == 0) +lean_dec(x_1); +x_36 = !lean_is_exclusive(x_20); +if (x_36 == 0) { -return x_15; +return x_20; } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_15, 0); -x_18 = lean_ctor_get(x_15, 1); -lean_inc(x_18); -lean_inc(x_17); -lean_dec(x_15); -x_19 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_19, 0, x_17); -lean_ctor_set(x_19, 1, x_18); -return x_19; +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_20, 0); +x_38 = lean_ctor_get(x_20, 1); +lean_inc(x_38); +lean_inc(x_37); +lean_dec(x_20); +x_39 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_39, 0, x_37); +lean_ctor_set(x_39, 1, x_38); +return x_39; } } -else +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: { -uint8_t x_20; -x_20 = !lean_is_exclusive(x_15); -if (x_20 == 0) +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; 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___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); +x_16 = lean_unsigned_to_nat(1u); +x_17 = lean_nat_sub(x_13, x_16); +lean_dec(x_13); +x_18 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_6, x_15, x_17); +x_19 = lean_box(0); +lean_inc(x_3); +lean_inc(x_2); +x_20 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__1(x_1, x_5, x_18, x_2, x_3, x_2, x_16, x_19, x_7, x_8, x_9, x_10, x_11); +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +x_22 = lean_array_get_size(x_5); +lean_inc(x_3); +x_23 = l_Array_toSubarray___rarg(x_5, x_3, x_22); +x_24 = lean_ctor_get(x_23, 2); +lean_inc(x_24); +x_25 = lean_usize_of_nat(x_24); +lean_dec(x_24); +x_26 = lean_ctor_get(x_23, 1); +lean_inc(x_26); +x_27 = lean_usize_of_nat(x_26); +lean_dec(x_26); +x_28 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__9(x_3, x_4, x_2, x_1, x_14, x_18, x_23, x_25, x_27, x_19, x_7, x_8, x_9, x_10, x_21); +lean_dec(x_23); +if (lean_obj_tag(x_28) == 0) { -return x_15; +uint8_t x_29; +x_29 = !lean_is_exclusive(x_28); +if (x_29 == 0) +{ +lean_object* x_30; +x_30 = lean_ctor_get(x_28, 0); +lean_dec(x_30); +lean_ctor_set(x_28, 0, x_19); +return x_28; } 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_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_19); +lean_ctor_set(x_32, 1, x_31); +return x_32; } } +else +{ +uint8_t x_33; +x_33 = !lean_is_exclusive(x_28); +if (x_33 == 0) +{ +return x_28; } else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_10, 1); -lean_inc(x_24); -lean_dec(x_10); -x_25 = lean_box(0); -x_26 = l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__5___lambda__1(x_1, x_2, x_25, x_3, x_4, x_5, x_6, x_7, x_8, x_24); -return x_26; +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_withSaveInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_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: { -lean_object* x_8; uint8_t x_9; -x_8 = l_Lean_Elab_CommandContextInfo_save___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -x_9 = !lean_is_exclusive(x_8); -if (x_9 == 0) +if (lean_obj_tag(x_5) == 0) { -lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_10 = lean_ctor_get(x_8, 0); -x_11 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_11, 0, x_10); -x_12 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_12, 0, x_11); -lean_ctor_set(x_8, 0, x_12); -return x_8; +lean_object* x_11; uint8_t x_12; +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_11 = lean_st_ref_get(x_4, x_10); +lean_dec(x_4); +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; lean_object* x_16; lean_object* x_17; -x_13 = lean_ctor_get(x_8, 0); -x_14 = lean_ctor_get(x_8, 1); +lean_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_8); -x_15 = lean_alloc_ctor(0, 1, 0); +lean_dec(x_11); +x_15 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_15, 0, x_13); -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_14); -return x_17; -} +lean_ctor_set(x_15, 1, x_14); +return x_15; } } -static lean_object* _init_l_Lean_Elab_withSaveInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__4___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_withSaveInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__4___lambda__1___boxed), 7, 0); -return x_1; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_withSaveInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; lean_object* x_21; +x_16 = lean_ctor_get(x_5, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_5, 1); +lean_inc(x_17); +lean_dec(x_5); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +lean_inc(x_2); +lean_inc(x_1); +lean_inc(x_3); +lean_inc(x_4); +x_19 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___lambda__1), 11, 4); +lean_closure_set(x_19, 0, x_4); +lean_closure_set(x_19, 1, x_3); +lean_closure_set(x_19, 2, x_1); +lean_closure_set(x_19, 3, x_2); +x_20 = 0; +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +x_21 = l_Lean_Meta_forallTelescopeReducing___at_Lean_Meta_getParamNames___spec__2___rarg(x_18, x_19, x_20, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_21) == 0) { -lean_object* x_9; lean_object* x_10; -x_9 = l_Lean_Elab_withSaveInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__4___closed__1; -x_10 = l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__5(x_1, x_9, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -return x_10; -} +lean_object* x_22; +x_22 = lean_ctor_get(x_21, 1); +lean_inc(x_22); +lean_dec(x_21); +x_5 = x_17; +x_10 = x_22; +goto _start; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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, 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) { -_start: -{ -lean_object* x_16; lean_object* x_17; -lean_inc(x_8); -x_16 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectLevelParamsInInductive(x_8); -x_17 = l_Lean_Elab_sortDeclLevelParams(x_1, x_2, x_16); -if (lean_obj_tag(x_17) == 0) +else { -uint8_t x_18; +uint8_t x_24; +lean_dec(x_17); +lean_dec(x_9); lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -x_18 = !lean_is_exclusive(x_17); -if (x_18 == 0) +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_24 = !lean_is_exclusive(x_21); +if (x_24 == 0) { -lean_object* x_19; lean_object* x_20; -lean_ctor_set_tag(x_17, 3); -x_19 = l_Lean_MessageData_ofFormat(x_17); -x_20 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_19, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -return x_20; +return x_21; } else { -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(3, 1, 0); -lean_ctor_set(x_22, 0, x_21); -x_23 = l_Lean_MessageData_ofFormat(x_22); -x_24 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_23, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -lean_dec(x_14); -lean_dec(x_13); +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_21, 0); +x_26 = lean_ctor_get(x_21, 1); +lean_inc(x_26); +lean_inc(x_25); +lean_dec(x_21); +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_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; +x_14 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); -return x_24; +lean_dec(x_9); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_14; } } -else +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: { -lean_object* x_25; lean_object* x_26; -x_25 = lean_ctor_get(x_17, 0); -lean_inc(x_25); -lean_dec(x_17); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_6); -lean_inc(x_25); -x_26 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts(x_3, x_4, x_25, x_5, x_6, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -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(6, 3, 1); -lean_ctor_set(x_29, 0, x_25); -lean_ctor_set(x_29, 1, x_6); -lean_ctor_set(x_29, 2, x_27); -lean_ctor_set_uint8(x_29, sizeof(void*)*3, x_7); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_29); -x_30 = l_Lean_Elab_Term_ensureNoUnassignedMVars(x_29, x_9, x_10, x_11, x_12, x_13, x_14, x_28); -if (lean_obj_tag(x_30) == 0) -{ -lean_object* x_31; lean_object* x_32; -x_31 = lean_ctor_get(x_30, 1); -lean_inc(x_31); -lean_dec(x_30); -lean_inc(x_14); -lean_inc(x_13); -x_32 = l_Lean_addDecl(x_29, x_13, x_14, x_31); -if (lean_obj_tag(x_32) == 0) -{ -lean_object* x_33; lean_object* x_34; -x_33 = lean_ctor_get(x_32, 1); -lean_inc(x_33); -lean_dec(x_32); -x_34 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions(x_3, x_9, x_10, x_11, x_12, x_13, x_14, x_33); -lean_dec(x_10); -lean_dec(x_9); -return x_34; +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_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___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; } -else +} +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___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) { +_start: { -uint8_t x_35; -lean_dec(x_14); +lean_object* x_15; +x_15 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___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); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); -lean_dec(x_9); -x_35 = !lean_is_exclusive(x_32); -if (x_35 == 0) -{ -return x_32; -} -else -{ -lean_object* x_36; lean_object* x_37; lean_object* x_38; -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_alloc_ctor(1, 2, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -return x_38; -} +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_15; } } -else +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___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) { +_start: { -uint8_t x_39; -lean_dec(x_29); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); +lean_object* x_12; +x_12 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_10); lean_dec(x_9); -x_39 = !lean_is_exclusive(x_30); -if (x_39 == 0) -{ -return x_30; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_1); +return x_12; } -else -{ -lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_40 = lean_ctor_get(x_30, 0); -x_41 = lean_ctor_get(x_30, 1); -lean_inc(x_41); -lean_inc(x_40); -lean_dec(x_30); -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_ForEachExprWhere_visited___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; +x_8 = l_Lean_ForEachExprWhere_visited___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__7(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_8; } } -else +LEAN_EXPORT lean_object* l_Lean_ForEachExprWhere_checked___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: { -uint8_t x_43; -lean_dec(x_25); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); +lean_object* x_8; +x_8 = l_Lean_ForEachExprWhere_checked___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_6); -x_43 = !lean_is_exclusive(x_26); -if (x_43 == 0) +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_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___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: { -return x_26; +uint8_t x_12; lean_object* x_13; +x_12 = lean_unbox(x_4); +lean_dec(x_4); +x_13 = l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6___lambda__1(x_1, x_2, x_3, x_12, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_6); +lean_dec(x_5); +return x_13; } -else +} +LEAN_EXPORT lean_object* l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_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: { -lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_44 = lean_ctor_get(x_26, 0); -x_45 = lean_ctor_get(x_26, 1); -lean_inc(x_45); -lean_inc(x_44); -lean_dec(x_26); -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; +uint8_t x_11; lean_object* x_12; +x_11 = lean_unbox(x_3); +lean_dec(x_3); +x_12 = l_Lean_ForEachExprWhere_visit_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__6(x_1, x_2, x_11, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_5); +return x_12; +} } +LEAN_EXPORT lean_object* l_Lean_ForEachExprWhere_visit___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___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_4); +lean_dec(x_4); +x_11 = l_Lean_ForEachExprWhere_visit___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__5(x_1, x_2, x_3, x_10, x_5, x_6, x_7, x_8, x_9); +return x_11; } } +LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__9___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +uint8_t x_3; lean_object* x_4; +x_3 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__9___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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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, uint8_t x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__9___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_array_get_size(x_9); -x_18 = lean_nat_add(x_17, x_1); -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_19 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateParams(x_9, x_2, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_19) == 0) +lean_object* x_12; +x_12 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__9___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +_start: { -if (lean_obj_tag(x_8) == 0) +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_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__9(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); +return x_18; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask(lean_object* x_1, lean_object* x_2, lean_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_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_19, 1); -lean_inc(x_21); -lean_dec(x_19); -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_20); -lean_inc(x_18); +lean_object* x_9; +lean_inc(x_7); +lean_inc(x_6); lean_inc(x_5); -x_22 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses(x_5, x_18, x_20, x_10, x_11, x_12, x_13, x_14, x_15, x_21); -if (lean_obj_tag(x_22) == 0) +lean_inc(x_4); +lean_inc(x_2); +x_9 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getArity(x_2, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_9) == 0) { -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_23 = lean_ctor_get(x_22, 1); +uint8_t x_10; +x_10 = !lean_is_exclusive(x_9); +if (x_10 == 0) +{ +lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_11 = lean_ctor_get(x_9, 0); +x_12 = lean_ctor_get(x_9, 1); +x_13 = lean_nat_dec_le(x_11, x_1); +if (x_13 == 0) +{ +uint8_t x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +lean_free_object(x_9); +x_14 = 0; +x_15 = lean_box(x_14); +lean_inc(x_1); +x_16 = lean_mk_array(x_1, x_15); +x_17 = lean_nat_sub(x_11, x_1); +x_18 = 1; +x_19 = lean_box(x_18); +x_20 = lean_mk_array(x_17, x_19); +x_21 = l_Array_append___rarg(x_16, x_20); +lean_dec(x_20); +x_22 = lean_st_mk_ref(x_21, x_12); +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_24 = lean_box(0); -x_25 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam(x_20, x_24, x_10, x_11, x_12, x_13, x_14, x_15, x_23); -x_26 = lean_ctor_get(x_25, 0); -lean_inc(x_26); -x_27 = lean_ctor_get(x_25, 1); -lean_inc(x_27); -lean_dec(x_25); -x_28 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__1(x_3, x_4, x_5, x_6, x_17, x_18, x_7, x_26, x_10, x_11, x_12, x_13, x_14, x_15, x_27); -lean_dec(x_5); -return x_28; +x_25 = lean_ctor_get(x_2, 2); +lean_inc(x_25); +lean_dec(x_2); +x_26 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go(x_1, x_3, x_11, x_23, x_25, x_4, x_5, x_6, x_7, x_24); +return x_26; } else { -uint8_t x_29; -lean_dec(x_20); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); +uint8_t x_27; lean_object* x_28; lean_object* x_29; +lean_dec(x_7); +lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_29 = !lean_is_exclusive(x_22); -if (x_29 == 0) -{ -return x_22; +lean_dec(x_2); +lean_dec(x_1); +x_27 = 0; +x_28 = lean_box(x_27); +x_29 = lean_mk_array(x_11, x_28); +lean_ctor_set(x_9, 0, x_29); +return x_9; +} } else { -lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_30 = lean_ctor_get(x_22, 0); -x_31 = lean_ctor_get(x_22, 1); +lean_object* x_30; lean_object* x_31; uint8_t x_32; +x_30 = lean_ctor_get(x_9, 0); +x_31 = lean_ctor_get(x_9, 1); lean_inc(x_31); lean_inc(x_30); -lean_dec(x_22); -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_9); +x_32 = lean_nat_dec_le(x_30, x_1); +if (x_32 == 0) +{ +uint8_t x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_33 = 0; +x_34 = lean_box(x_33); +lean_inc(x_1); +x_35 = lean_mk_array(x_1, x_34); +x_36 = lean_nat_sub(x_30, x_1); +x_37 = 1; +x_38 = lean_box(x_37); +x_39 = lean_mk_array(x_36, x_38); +x_40 = l_Array_append___rarg(x_35, x_39); +lean_dec(x_39); +x_41 = lean_st_mk_ref(x_40, x_31); +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_2, 2); +lean_inc(x_44); +lean_dec(x_2); +x_45 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go(x_1, x_3, x_30, x_42, x_44, x_4, x_5, x_6, x_7, x_43); +return x_45; } else { -lean_object* x_33; lean_object* x_34; uint8_t x_35; -x_33 = lean_ctor_get(x_19, 0); -lean_inc(x_33); -x_34 = lean_ctor_get(x_19, 1); -lean_inc(x_34); -lean_dec(x_19); -x_35 = !lean_is_exclusive(x_8); -if (x_35 == 0) -{ -lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_36 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam(x_33, x_8, x_10, x_11, x_12, x_13, x_14, x_15, x_34); -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_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_18); -x_39 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse(x_5, x_18, x_37, x_10, x_11, x_12, x_13, x_14, x_15, x_38); -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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__1(x_3, x_4, x_5, x_6, x_17, x_18, x_7, x_40, x_10, x_11, x_12, x_13, x_14, x_15, x_41); +uint8_t x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; +lean_dec(x_7); +lean_dec(x_6); lean_dec(x_5); -return x_42; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_46 = 0; +x_47 = lean_box(x_46); +x_48 = lean_mk_array(x_30, x_47); +x_49 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_49, 0, x_48); +lean_ctor_set(x_49, 1, x_31); +return x_49; +} +} } else { -uint8_t x_43; -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); +uint8_t x_50; +lean_dec(x_7); +lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_43 = !lean_is_exclusive(x_39); -if (x_43 == 0) +lean_dec(x_2); +lean_dec(x_1); +x_50 = !lean_is_exclusive(x_9); +if (x_50 == 0) { -return x_39; +return x_9; } else { -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; +lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_51 = lean_ctor_get(x_9, 0); +x_52 = lean_ctor_get(x_9, 1); +lean_inc(x_52); +lean_inc(x_51); +lean_dec(x_9); +x_53 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_53, 0, x_51); +lean_ctor_set(x_53, 1, x_52); +return x_53; } } } -else +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isDomainDefEq(lean_object* x_1, 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_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_47 = lean_ctor_get(x_8, 0); -lean_inc(x_47); -lean_dec(x_8); -x_48 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_48, 0, x_47); -x_49 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam(x_33, x_48, x_10, x_11, x_12, x_13, x_14, x_15, x_34); -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_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_18); -x_52 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse(x_5, x_18, x_50, x_10, x_11, x_12, x_13, x_14, x_15, x_51); -if (lean_obj_tag(x_52) == 0) +uint8_t x_8; +x_8 = l_Lean_Expr_isForall(x_1); +if (x_8 == 0) { -lean_object* x_53; lean_object* x_54; lean_object* x_55; -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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__1(x_3, x_4, x_5, x_6, x_17, x_18, x_7, x_53, x_10, x_11, x_12, x_13, x_14, x_15, x_54); +uint8_t x_9; lean_object* x_10; lean_object* x_11; +lean_dec(x_6); lean_dec(x_5); -return x_55; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_9 = 0; +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; } else { -lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_56 = lean_ctor_get(x_52, 0); -lean_inc(x_56); -x_57 = lean_ctor_get(x_52, 1); -lean_inc(x_57); -if (lean_is_exclusive(x_52)) { - lean_ctor_release(x_52, 0); - lean_ctor_release(x_52, 1); - x_58 = x_52; -} else { - lean_dec_ref(x_52); - x_58 = lean_box(0); -} -if (lean_is_scalar(x_58)) { - x_59 = lean_alloc_ctor(1, 2, 0); -} else { - x_59 = x_58; +lean_object* x_12; lean_object* x_13; +x_12 = l_Lean_Expr_bindingDomain_x21(x_1); +x_13 = l_Lean_Meta_isExprDefEq(x_12, x_2, x_3, x_4, x_5, x_6, x_7); +return x_13; } -lean_ctor_set(x_59, 0, x_56); -lean_ctor_set(x_59, 1, x_57); -return x_59; } } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isDomainDefEq___boxed(lean_object* x_1, 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_Inductive_0__Lean_Elab_Command_isDomainDefEq(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_1); +return x_8; } } -else +LEAN_EXPORT lean_object* l_List_allM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_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: { -uint8_t x_60; -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_8); +if (lean_obj_tag(x_2) == 0) +{ +uint8_t x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_60 = !lean_is_exclusive(x_19); -if (x_60 == 0) -{ -return x_19; +lean_dec(x_1); +x_8 = 1; +x_9 = lean_box(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_7); +return x_10; } else { -lean_object* x_61; lean_object* x_62; lean_object* x_63; -x_61 = lean_ctor_get(x_19, 0); -x_62 = lean_ctor_get(x_19, 1); -lean_inc(x_62); -lean_inc(x_61); -lean_dec(x_19); -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; -} -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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, uint8_t x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_2, 0); +x_12 = lean_ctor_get(x_2, 1); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_1); +x_13 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isDomainDefEq(x_11, x_1, x_3, x_4, x_5, x_6, x_7); +if (lean_obj_tag(x_13) == 0) { -lean_object* x_17; lean_object* x_18; -x_17 = lean_array_to_list(x_1); -lean_inc(x_15); +lean_object* x_14; uint8_t x_15; +x_14 = lean_ctor_get(x_13, 0); lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_17); -x_18 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse(x_17, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_18) == 0) -{ -lean_object* x_19; lean_object* x_20; lean_object* x_21; -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); -x_21 = l_Lean_Elab_Command_shouldInferResultUniverse(x_19, x_10, x_11, x_12, x_13, x_14, x_15, x_20); -if (lean_obj_tag(x_21) == 0) -{ -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; 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_box(x_7); -lean_inc(x_17); -x_25 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__2___boxed), 16, 8); -lean_closure_set(x_25, 0, x_2); -lean_closure_set(x_25, 1, x_17); -lean_closure_set(x_25, 2, x_3); -lean_closure_set(x_25, 3, x_4); -lean_closure_set(x_25, 4, x_5); -lean_closure_set(x_25, 5, x_6); -lean_closure_set(x_25, 6, x_24); -lean_closure_set(x_25, 7, x_22); -x_26 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withUsed___rarg(x_8, x_17, x_25, x_10, x_11, x_12, x_13, x_14, x_15, x_23); -return x_26; -} -else -{ -uint8_t x_27; -lean_dec(x_17); -lean_dec(x_15); +x_15 = lean_unbox(x_14); lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); +if (x_15 == 0) +{ +uint8_t x_16; 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_21); -if (x_27 == 0) +lean_dec(x_1); +x_16 = !lean_is_exclusive(x_13); +if (x_16 == 0) { -return x_21; +lean_object* x_17; uint8_t x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_13, 0); +lean_dec(x_17); +x_18 = 0; +x_19 = lean_box(x_18); +lean_ctor_set(x_13, 0, x_19); +return x_13; } 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_20; uint8_t x_21; lean_object* x_22; lean_object* x_23; +x_20 = lean_ctor_get(x_13, 1); +lean_inc(x_20); +lean_dec(x_13); +x_21 = 0; +x_22 = lean_box(x_21); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_20); +return x_23; } } else { -uint8_t x_31; -lean_dec(x_17); -lean_dec(x_15); -lean_dec(x_14); +lean_object* x_24; +x_24 = lean_ctor_get(x_13, 1); +lean_inc(x_24); lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); +x_2 = x_12; +x_7 = x_24; +goto _start; +} +} +else +{ +uint8_t x_26; lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); -x_31 = !lean_is_exclusive(x_18); -if (x_31 == 0) +lean_dec(x_1); +x_26 = !lean_is_exclusive(x_13); +if (x_26 == 0) { -return x_18; +return x_13; } else { -lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_32 = lean_ctor_get(x_18, 0); -x_33 = lean_ctor_get(x_18, 1); -lean_inc(x_33); -lean_inc(x_32); -lean_dec(x_18); -x_34 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_34, 0, x_32); -lean_ctor_set(x_34, 1, x_33); -return x_34; -} -} -} +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; } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__4___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("numExplicitParams: ", 19, 19); -return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__4___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__4___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, uint8_t x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_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_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___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_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_18 = lean_array_get_size(x_1); -x_19 = lean_unsigned_to_nat(0u); -x_20 = lean_unsigned_to_nat(1u); -x_21 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__3___closed__1; -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_18); -lean_inc(x_4); -lean_inc(x_3); -x_22 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__1(x_1, x_2, x_3, x_4, x_18, x_18, x_19, x_18, x_20, x_21, x_11, x_12, x_13, x_14, x_15, x_16, x_17); -lean_dec(x_18); -if (lean_obj_tag(x_22) == 0) -{ -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -x_24 = lean_ctor_get(x_22, 1); -lean_inc(x_24); -lean_dec(x_22); -x_25 = lean_array_get_size(x_3); -lean_dec(x_3); -lean_inc(x_16); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_4); -lean_inc(x_23); -x_26 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams(x_25, x_23, x_4, x_13, x_14, x_15, x_16, x_24); -if (lean_obj_tag(x_26) == 0) -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; -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_5); -x_29 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_5, x_11, x_12, x_13, x_14, x_15, x_16, x_28); -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) +if (lean_obj_tag(x_2) == 0) { -lean_object* x_32; lean_object* x_33; lean_object* x_34; +lean_object* x_9; lean_object* x_10; +lean_dec(x_7); +lean_dec(x_6); lean_dec(x_5); -x_32 = lean_ctor_get(x_29, 1); -lean_inc(x_32); -lean_dec(x_29); -x_33 = lean_box(0); -x_34 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__3(x_23, x_27, x_6, x_7, x_1, x_4, x_8, x_9, x_33, x_11, x_12, x_13, x_14, x_15, x_16, x_32); -return x_34; +lean_dec(x_4); +x_9 = l_List_reverse___rarg(x_3); +x_10 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set(x_10, 1, x_8); +return x_10; } else { -uint8_t x_35; -x_35 = !lean_is_exclusive(x_29); -if (x_35 == 0) +uint8_t x_11; +x_11 = !lean_is_exclusive(x_2); +if (x_11 == 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; -x_36 = lean_ctor_get(x_29, 1); -x_37 = lean_ctor_get(x_29, 0); -lean_dec(x_37); -lean_inc(x_27); -x_38 = l___private_Init_Data_Repr_0__Nat_reprFast(x_27); -x_39 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_39, 0, x_38); -x_40 = l_Lean_MessageData_ofFormat(x_39); -x_41 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__4___closed__2; -lean_ctor_set_tag(x_29, 7); -lean_ctor_set(x_29, 1, x_40); -lean_ctor_set(x_29, 0, x_41); -x_42 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5; -x_43 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_43, 0, x_29); -lean_ctor_set(x_43, 1, x_42); -x_44 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_5, x_43, x_11, x_12, x_13, x_14, x_15, x_16, x_36); -x_45 = lean_ctor_get(x_44, 0); -lean_inc(x_45); -x_46 = lean_ctor_get(x_44, 1); -lean_inc(x_46); -lean_dec(x_44); -x_47 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__3(x_23, x_27, x_6, x_7, x_1, x_4, x_8, x_9, x_45, x_11, x_12, x_13, x_14, x_15, x_16, x_46); -lean_dec(x_45); -return x_47; -} -else +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_12 = lean_ctor_get(x_2, 0); +x_13 = lean_ctor_get(x_2, 1); +x_14 = l_Lean_Expr_bindingBody_x21(x_12); +lean_dec(x_12); +x_15 = lean_expr_instantiate1(x_14, x_1); +lean_dec(x_14); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_16 = l_Lean_Meta_whnfD(x_15, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_16) == 0) { -lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; -x_48 = lean_ctor_get(x_29, 1); -lean_inc(x_48); -lean_dec(x_29); -lean_inc(x_27); -x_49 = l___private_Init_Data_Repr_0__Nat_reprFast(x_27); -x_50 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_50, 0, x_49); -x_51 = l_Lean_MessageData_ofFormat(x_50); -x_52 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__4___closed__2; -x_53 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_53, 0, x_52); -lean_ctor_set(x_53, 1, x_51); -x_54 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5; -x_55 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_55, 0, x_53); -lean_ctor_set(x_55, 1, x_54); -x_56 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_5, x_55, x_11, x_12, x_13, x_14, x_15, x_16, x_48); -x_57 = lean_ctor_get(x_56, 0); -lean_inc(x_57); -x_58 = lean_ctor_get(x_56, 1); -lean_inc(x_58); -lean_dec(x_56); -x_59 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__3(x_23, x_27, x_6, x_7, x_1, x_4, x_8, x_9, x_57, x_11, x_12, x_13, x_14, x_15, x_16, x_58); -lean_dec(x_57); -return x_59; -} +lean_object* x_17; lean_object* x_18; +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_2, 1, x_3); +lean_ctor_set(x_2, 0, x_17); +{ +lean_object* _tmp_1 = x_13; +lean_object* _tmp_2 = x_2; +lean_object* _tmp_7 = x_18; +x_2 = _tmp_1; +x_3 = _tmp_2; +x_8 = _tmp_7; } +goto _start; } else { -uint8_t x_60; -lean_dec(x_23); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); +uint8_t x_20; +lean_free_object(x_2); lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_1); -x_60 = !lean_is_exclusive(x_26); -if (x_60 == 0) +lean_dec(x_3); +x_20 = !lean_is_exclusive(x_16); +if (x_20 == 0) { -return x_26; +return x_16; } else { -lean_object* x_61; lean_object* x_62; lean_object* x_63; -x_61 = lean_ctor_get(x_26, 0); -x_62 = lean_ctor_get(x_26, 1); -lean_inc(x_62); -lean_inc(x_61); -lean_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); -return x_63; +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 { -uint8_t x_64; -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_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_24 = lean_ctor_get(x_2, 0); +x_25 = lean_ctor_get(x_2, 1); +lean_inc(x_25); +lean_inc(x_24); +lean_dec(x_2); +x_26 = l_Lean_Expr_bindingBody_x21(x_24); +lean_dec(x_24); +x_27 = lean_expr_instantiate1(x_26, x_1); +lean_dec(x_26); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_28 = l_Lean_Meta_whnfD(x_27, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_28) == 0) +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_28, 0); +lean_inc(x_29); +x_30 = lean_ctor_get(x_28, 1); +lean_inc(x_30); +lean_dec(x_28); +x_31 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_31, 0, x_29); +lean_ctor_set(x_31, 1, x_3); +x_2 = x_25; +x_3 = x_31; +x_8 = x_30; +goto _start; +} +else +{ +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; +lean_dec(x_25); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_1); -x_64 = !lean_is_exclusive(x_22); -if (x_64 == 0) -{ -return x_22; -} -else -{ -lean_object* x_65; lean_object* x_66; lean_object* x_67; -x_65 = lean_ctor_get(x_22, 0); -x_66 = lean_ctor_get(x_22, 1); -lean_inc(x_66); -lean_inc(x_65); -lean_dec(x_22); -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_33 = lean_ctor_get(x_28, 0); +lean_inc(x_33); +x_34 = lean_ctor_get(x_28, 1); +lean_inc(x_34); +if (lean_is_exclusive(x_28)) { + lean_ctor_release(x_28, 0); + lean_ctor_release(x_28, 1); + x_35 = x_28; +} else { + lean_dec_ref(x_28); + x_35 = lean_box(0); } +if (lean_is_scalar(x_35)) { + x_36 = lean_alloc_ctor(1, 2, 0); +} else { + x_36 = x_35; } +lean_ctor_set(x_36, 0, x_33); +lean_ctor_set(x_36, 1, x_34); +return x_36; } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__5___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("indFVars: ", 10, 10); -return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__5___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__5___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__5(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_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___spec__3(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4) { _start: { -lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; -x_16 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__3; -x_17 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_16, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -x_19 = lean_unbox(x_18); -lean_dec(x_18); -if (x_19 == 0) +uint8_t x_5; +x_5 = lean_usize_dec_eq(x_3, x_4); +if (x_5 == 0) { -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_17, 1); -lean_inc(x_20); -lean_dec(x_17); -x_21 = lean_box(0); -x_22 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__4(x_1, x_2, x_7, x_8, x_16, x_3, x_4, x_5, x_6, x_21, x_9, x_10, x_11, x_12, x_13, x_14, x_20); -return x_22; -} -else +lean_object* x_6; lean_object* x_7; uint8_t x_8; +x_6 = lean_array_uget(x_2, x_3); +x_7 = lean_array_get_size(x_6); +x_8 = lean_nat_dec_lt(x_1, x_7); +lean_dec(x_7); +if (x_8 == 0) { -uint8_t x_23; -x_23 = !lean_is_exclusive(x_17); -if (x_23 == 0) +uint8_t x_9; +lean_dec(x_6); +x_9 = 1; +return x_9; +} +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_17, 1); -x_25 = lean_ctor_get(x_17, 0); -lean_dec(x_25); -lean_inc(x_8); -x_26 = lean_array_to_list(x_8); -x_27 = lean_box(0); -x_28 = l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(x_26, x_27); -x_29 = l_Lean_MessageData_ofList(x_28); -x_30 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__5___closed__2; -lean_ctor_set_tag(x_17, 7); -lean_ctor_set(x_17, 1, x_29); -lean_ctor_set(x_17, 0, x_30); -x_31 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5; -x_32 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_32, 0, x_17); -lean_ctor_set(x_32, 1, x_31); -x_33 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_16, x_32, x_9, x_10, x_11, x_12, x_13, x_14, x_24); -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_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__4(x_1, x_2, x_7, x_8, x_16, x_3, x_4, x_5, x_6, x_34, x_9, x_10, x_11, x_12, x_13, x_14, x_35); -lean_dec(x_34); -return x_36; +lean_object* x_10; uint8_t x_11; +x_10 = lean_array_fget(x_6, x_1); +lean_dec(x_6); +x_11 = lean_unbox(x_10); +lean_dec(x_10); +if (x_11 == 0) +{ +uint8_t x_12; +x_12 = 1; +return x_12; } 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_17, 1); -lean_inc(x_37); -lean_dec(x_17); -lean_inc(x_8); -x_38 = lean_array_to_list(x_8); -x_39 = lean_box(0); -x_40 = l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(x_38, x_39); -x_41 = l_Lean_MessageData_ofList(x_40); -x_42 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__5___closed__2; -x_43 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_43, 0, x_42); -lean_ctor_set(x_43, 1, x_41); -x_44 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5; -x_45 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_45, 0, x_43); -lean_ctor_set(x_45, 1, x_44); -x_46 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_16, x_45, x_9, x_10, x_11, x_12, x_13, x_14, x_37); -x_47 = lean_ctor_get(x_46, 0); -lean_inc(x_47); -x_48 = lean_ctor_get(x_46, 1); -lean_inc(x_48); -lean_dec(x_46); -x_49 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__4(x_1, x_2, x_7, x_8, x_16, x_3, x_4, x_5, x_6, x_47, x_9, x_10, x_11, x_12, x_13, x_14, x_48); -lean_dec(x_47); -return x_49; +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 = 0; +return x_16; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__6(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_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_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) { _start: { -lean_object* x_11; lean_object* x_12; -x_11 = lean_box(0); -x_12 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__3(x_1, x_2, x_3, 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_8; +x_8 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_8, 0, x_1); +lean_ctor_set(x_8, 1, x_7); +return x_8; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_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) { +_start: { -uint8_t x_13; -x_13 = !lean_is_exclusive(x_12); -if (x_13 == 0) +lean_object* x_12; lean_object* x_13; +x_12 = lean_box(0); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +x_13 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___spec__2(x_6, x_1, x_12, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_13) == 0) { -lean_object* x_14; -x_14 = lean_ctor_get(x_12, 0); -lean_dec(x_14); -lean_ctor_set(x_12, 0, x_11); -return x_12; +lean_object* x_14; 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_inc(x_15); +lean_dec(x_13); +x_16 = lean_unsigned_to_nat(1u); +x_17 = lean_nat_add(x_2, x_16); +x_18 = l_Lean_Expr_bindingBody_x21(x_3); +x_19 = lean_expr_instantiate1(x_18, x_6); +lean_dec(x_18); +x_20 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go(x_4, x_5, x_17, x_19, x_14, x_7, x_8, x_9, x_10, x_15); +return x_20; } else { -lean_object* x_15; lean_object* x_16; -x_15 = lean_ctor_get(x_12, 1); -lean_inc(x_15); -lean_dec(x_12); -x_16 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_16, 0, x_11); -lean_ctor_set(x_16, 1, x_15); -return x_16; -} +uint8_t x_21; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_4); +x_21 = !lean_is_exclusive(x_13); +if (x_21 == 0) +{ +return x_13; } else { -uint8_t x_17; -x_17 = !lean_is_exclusive(x_12); -if (x_17 == 0) +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_13, 0); +x_23 = lean_ctor_get(x_13, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_13); +x_24 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); +return x_24; +} +} +} +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__3___closed__1() { +_start: { -return x_12; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("a", 1, 1); +return x_1; } -else +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__3___closed__2() { +_start: { -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_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__3___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_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) { +_start: +{ +lean_object* x_13; lean_object* x_14; uint8_t x_15; uint8_t x_16; lean_object* x_17; +x_13 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__2___boxed), 11, 5); +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); +x_14 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__3___closed__2; +x_15 = 0; +x_16 = 0; +x_17 = l_Lean_Meta_withLocalDecl___at_Lean_Meta_forallTelescopeCompatibleAux___spec__15___rarg(x_14, x_15, x_6, x_13, x_16, x_8, x_9, x_10, x_11, x_12); +return x_17; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__7___boxed__const__1() { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4___closed__1() { _start: { -size_t x_1; lean_object* x_2; -x_1 = 0; -x_2 = lean_box_usize(x_1); +lean_object* x_1; +x_1 = lean_mk_string_unchecked("domain not def eq: ", 19, 19); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4___closed__3() { _start: { -lean_object* x_13; -lean_inc(x_11); +lean_object* x_1; +x_1 = lean_mk_string_unchecked(", ", 2, 2); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" =\?= ", 5, 5); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4___closed__5; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; lean_object* x_13; +x_12 = l_Lean_Expr_bindingDomain_x21(x_1); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_1); -x_13 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeader(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_inc(x_12); +x_13 = l_List_allM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___spec__1(x_12, x_2, x_7, x_8, x_9, x_10, x_11); if (lean_obj_tag(x_13) == 0) { -lean_object* x_14; lean_object* x_15; uint8_t x_16; uint8_t x_17; lean_object* x_18; +lean_object* x_14; uint8_t x_15; x_14 = lean_ctor_get(x_13, 0); lean_inc(x_14); -x_15 = lean_ctor_get(x_13, 1); -lean_inc(x_15); -lean_dec(x_13); -x_16 = 1; -x_17 = 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_18 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_16, x_17, x_6, x_7, x_8, x_9, x_10, x_11, x_15); -if (lean_obj_tag(x_18) == 0) +x_15 = lean_unbox(x_14); +lean_dec(x_14); +if (x_15 == 0) { -lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_19 = lean_ctor_get(x_18, 1); +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +x_16 = lean_ctor_get(x_13, 1); +lean_inc(x_16); +lean_dec(x_13); +x_17 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__3; +x_18 = l_Lean_isTracingEnabledFor___at_Lean_Meta_processPostponed_loop___spec__1(x_17, x_7, x_8, x_9, x_10, x_16); +x_19 = lean_ctor_get(x_18, 0); lean_inc(x_19); -lean_dec(x_18); -x_20 = lean_box(x_4); -lean_inc(x_14); -lean_inc(x_1); -x_21 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__5___boxed), 15, 6); -lean_closure_set(x_21, 0, x_1); -lean_closure_set(x_21, 1, x_14); -lean_closure_set(x_21, 2, x_2); -lean_closure_set(x_21, 3, x_3); -lean_closure_set(x_21, 4, x_20); -lean_closure_set(x_21, 5, x_5); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -x_22 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls___rarg(x_14, x_21, x_6, x_7, x_8, x_9, x_10, x_11, x_19); -if (lean_obj_tag(x_22) == 0) +x_20 = lean_unbox(x_19); +lean_dec(x_19); +if (x_20 == 0) { -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; -x_23 = lean_ctor_get(x_22, 1); -lean_inc(x_23); +uint8_t x_21; +lean_dec(x_12); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_1); +x_21 = !lean_is_exclusive(x_18); +if (x_21 == 0) +{ +lean_object* x_22; +x_22 = lean_ctor_get(x_18, 0); lean_dec(x_22); -x_24 = lean_array_size(x_1); -x_25 = lean_box_usize(x_24); -x_26 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__7___boxed__const__1; -x_27 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__6___boxed), 10, 3); -lean_closure_set(x_27, 0, x_1); -lean_closure_set(x_27, 1, x_25); -lean_closure_set(x_27, 2, x_26); -x_28 = lean_alloc_closure((void*)(l_Lean_Elab_withSaveInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__4___lambda__1___boxed), 7, 0); -x_29 = l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__5(x_27, x_28, x_6, x_7, x_8, x_9, x_10, x_11, x_23); -return x_29; +lean_ctor_set(x_18, 0, x_3); +return x_18; } else { -uint8_t x_30; -lean_dec(x_11); +lean_object* x_23; lean_object* x_24; +x_23 = lean_ctor_get(x_18, 1); +lean_inc(x_23); +lean_dec(x_18); +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_3); +lean_ctor_set(x_24, 1, x_23); +return x_24; +} +} +else +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; +x_25 = lean_ctor_get(x_18, 1); +lean_inc(x_25); +lean_dec(x_18); +lean_inc(x_3); +x_26 = l___private_Init_Data_Repr_0__Nat_reprFast(x_3); +x_27 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_27, 0, x_26); +x_28 = l_Lean_MessageData_ofFormat(x_27); +x_29 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4___closed__2; +x_30 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_30, 0, x_29); +lean_ctor_set(x_30, 1, x_28); +x_31 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4___closed__4; +x_32 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_31); +x_33 = l_Lean_MessageData_ofExpr(x_1); +x_34 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_34, 0, x_32); +lean_ctor_set(x_34, 1, x_33); +x_35 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4___closed__6; +x_36 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_36, 0, x_34); +lean_ctor_set(x_36, 1, x_35); +x_37 = l_Lean_MessageData_ofExpr(x_12); +x_38 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_38, 0, x_36); +lean_ctor_set(x_38, 1, x_37); +x_39 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +x_40 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +x_41 = l_Lean_addTrace___at_Lean_Meta_processPostponed_loop___spec__2(x_17, x_40, x_7, x_8, x_9, x_10, 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_1); -x_30 = !lean_is_exclusive(x_22); -if (x_30 == 0) +x_42 = !lean_is_exclusive(x_41); +if (x_42 == 0) { -return x_22; +lean_object* x_43; +x_43 = lean_ctor_get(x_41, 0); +lean_dec(x_43); +lean_ctor_set(x_41, 0, x_3); +return x_41; } else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_31 = lean_ctor_get(x_22, 0); -x_32 = lean_ctor_get(x_22, 1); -lean_inc(x_32); -lean_inc(x_31); -lean_dec(x_22); -x_33 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_33, 0, x_31); -lean_ctor_set(x_33, 1, x_32); -return x_33; +lean_object* x_44; lean_object* x_45; +x_44 = lean_ctor_get(x_41, 1); +lean_inc(x_44); +lean_dec(x_41); +x_45 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_45, 0, x_3); +lean_ctor_set(x_45, 1, x_44); +return x_45; } } } else { -uint8_t x_34; -lean_dec(x_14); -lean_dec(x_11); +lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_46 = lean_ctor_get(x_13, 1); +lean_inc(x_46); +lean_dec(x_13); +x_47 = lean_box(0); +x_48 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__3(x_2, x_3, x_1, x_4, x_5, x_12, x_47, x_7, x_8, x_9, x_10, x_46); +return x_48; +} +} +else +{ +uint8_t x_49; +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); lean_dec(x_2); lean_dec(x_1); -x_34 = !lean_is_exclusive(x_18); -if (x_34 == 0) +x_49 = !lean_is_exclusive(x_13); +if (x_49 == 0) { -return x_18; +return x_13; } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_35 = lean_ctor_get(x_18, 0); -x_36 = lean_ctor_get(x_18, 1); -lean_inc(x_36); -lean_inc(x_35); -lean_dec(x_18); -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_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_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; } } } -else +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: { -uint8_t x_38; -lean_dec(x_11); +uint8_t x_12; +x_12 = l_Lean_Expr_isForall(x_1); +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); -lean_dec(x_3); +lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_38 = !lean_is_exclusive(x_13); -if (x_38 == 0) -{ +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_3); +lean_ctor_set(x_13, 1, x_11); return x_13; } else { -lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_39 = lean_ctor_get(x_13, 0); -x_40 = lean_ctor_get(x_13, 1); -lean_inc(x_40); -lean_inc(x_39); -lean_dec(x_13); -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_14; lean_object* x_15; +x_14 = lean_box(0); +x_15 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4(x_1, x_2, x_3, x_4, x_5, x_14, x_7, x_8, x_9, x_10, x_11); +return x_15; } } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_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: { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -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_object* x_11; uint8_t x_12; +x_11 = lean_array_get_size(x_2); +x_12 = lean_nat_dec_lt(x_3, x_11); lean_dec(x_11); -lean_inc(x_8); -lean_inc(x_4); -x_14 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkLevelNames(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_13); -if (lean_obj_tag(x_14) == 0) +if (x_12 == 0) { -lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; -x_15 = lean_ctor_get(x_14, 1); -lean_inc(x_15); -lean_dec(x_14); -x_16 = lean_ctor_get(x_2, 5); -lean_inc(x_16); -x_17 = lean_ctor_get(x_2, 2); -lean_inc(x_17); -x_18 = lean_ctor_get_uint8(x_17, sizeof(void*)*2 + 3); -lean_dec(x_17); -x_19 = lean_ctor_get(x_2, 0); -lean_inc(x_19); +lean_object* x_13; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); lean_dec(x_2); -x_20 = lean_box(x_18); -lean_inc(x_16); -x_21 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__7___boxed), 12, 5); -lean_closure_set(x_21, 0, x_1); -lean_closure_set(x_21, 1, x_12); -lean_closure_set(x_21, 2, x_16); -lean_closure_set(x_21, 3, x_20); -lean_closure_set(x_21, 4, x_3); -x_22 = !lean_is_exclusive(x_8); -if (x_22 == 0) -{ -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_8, 5); -x_24 = l_Lean_replaceRef(x_19, x_23); -lean_dec(x_23); -lean_dec(x_19); -lean_ctor_set(x_8, 5, x_24); -x_25 = l_Lean_Elab_Term_withLevelNames___rarg(x_16, x_21, x_4, x_5, x_6, x_7, x_8, x_9, x_15); -return x_25; +lean_dec(x_1); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_3); +lean_ctor_set(x_13, 1, x_10); +return x_13; } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; lean_object* x_38; uint8_t x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_26 = lean_ctor_get(x_8, 0); -x_27 = lean_ctor_get(x_8, 1); -x_28 = lean_ctor_get(x_8, 2); -x_29 = lean_ctor_get(x_8, 3); -x_30 = lean_ctor_get(x_8, 4); -x_31 = lean_ctor_get(x_8, 5); -x_32 = lean_ctor_get(x_8, 6); -x_33 = lean_ctor_get(x_8, 7); -x_34 = lean_ctor_get(x_8, 8); -x_35 = lean_ctor_get(x_8, 9); -x_36 = lean_ctor_get(x_8, 10); -x_37 = lean_ctor_get_uint8(x_8, sizeof(void*)*12); -x_38 = lean_ctor_get(x_8, 11); -x_39 = lean_ctor_get_uint8(x_8, sizeof(void*)*12 + 1); -lean_inc(x_38); -lean_inc(x_36); -lean_inc(x_35); -lean_inc(x_34); -lean_inc(x_33); -lean_inc(x_32); -lean_inc(x_31); -lean_inc(x_30); -lean_inc(x_29); -lean_inc(x_28); -lean_inc(x_27); -lean_inc(x_26); -lean_dec(x_8); -x_40 = l_Lean_replaceRef(x_19, x_31); -lean_dec(x_31); -lean_dec(x_19); -x_41 = lean_alloc_ctor(0, 12, 2); -lean_ctor_set(x_41, 0, x_26); -lean_ctor_set(x_41, 1, x_27); -lean_ctor_set(x_41, 2, x_28); -lean_ctor_set(x_41, 3, x_29); -lean_ctor_set(x_41, 4, x_30); -lean_ctor_set(x_41, 5, x_40); -lean_ctor_set(x_41, 6, x_32); -lean_ctor_set(x_41, 7, x_33); -lean_ctor_set(x_41, 8, x_34); -lean_ctor_set(x_41, 9, x_35); -lean_ctor_set(x_41, 10, x_36); -lean_ctor_set(x_41, 11, x_38); -lean_ctor_set_uint8(x_41, sizeof(void*)*12, x_37); -lean_ctor_set_uint8(x_41, sizeof(void*)*12 + 1, x_39); -x_42 = l_Lean_Elab_Term_withLevelNames___rarg(x_16, x_21, x_4, x_5, x_6, x_7, x_41, x_9, x_15); -return x_42; -} -} -else -{ -uint8_t x_43; -lean_dec(x_12); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_43 = !lean_is_exclusive(x_14); -if (x_43 == 0) +lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_14 = lean_array_get_size(x_1); +x_15 = lean_unsigned_to_nat(0u); +x_16 = lean_nat_dec_lt(x_15, x_14); +if (x_16 == 0) { -return x_14; +lean_object* x_17; lean_object* x_18; +lean_dec(x_14); +x_17 = lean_box(0); +x_18 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__5(x_4, x_5, x_3, x_1, x_2, x_17, x_6, x_7, x_8, x_9, x_10); +return x_18; } else { -lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_44 = lean_ctor_get(x_14, 0); -x_45 = lean_ctor_get(x_14, 1); -lean_inc(x_45); -lean_inc(x_44); +size_t x_19; size_t x_20; uint8_t x_21; +x_19 = 0; +x_20 = lean_usize_of_nat(x_14); lean_dec(x_14); -x_46 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_46, 0, x_44); -lean_ctor_set(x_46, 1, x_45); -return x_46; -} -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_10 = lean_array_get_size(x_2); -x_11 = lean_unsigned_to_nat(0u); -x_12 = lean_nat_dec_lt(x_11, x_10); -lean_dec(x_10); -if (x_12 == 0) +x_21 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___spec__3(x_3, x_1, x_19, x_20); +if (x_21 == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_13 = l_Lean_Elab_Command_instInhabitedInductiveView; -x_14 = l_outOfBounds___rarg(x_13); -x_15 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__8), 10, 3); -lean_closure_set(x_15, 0, x_2); -lean_closure_set(x_15, 1, x_14); -lean_closure_set(x_15, 2, x_1); -x_16 = l_Lean_Elab_Term_withoutSavingRecAppSyntax___rarg(x_15, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_16; +lean_object* x_22; lean_object* x_23; +x_22 = lean_box(0); +x_23 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__5(x_4, x_5, x_3, x_1, x_2, x_22, x_6, x_7, x_8, x_9, x_10); +return x_23; } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_array_fget(x_2, x_11); -x_18 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__8), 10, 3); -lean_closure_set(x_18, 0, x_2); -lean_closure_set(x_18, 1, x_17); -lean_closure_set(x_18, 2, x_1); -x_19 = l_Lean_Elab_Term_withoutSavingRecAppSyntax___rarg(x_18, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_19; -} -} -} -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__1___boxed(lean_object** _args) { -lean_object* x_1 = _args[0]; -lean_object* x_2 = _args[1]; -lean_object* x_3 = _args[2]; -lean_object* x_4 = _args[3]; -lean_object* x_5 = _args[4]; -lean_object* x_6 = _args[5]; -lean_object* x_7 = _args[6]; -lean_object* x_8 = _args[7]; -lean_object* x_9 = _args[8]; -lean_object* x_10 = _args[9]; -lean_object* x_11 = _args[10]; -lean_object* x_12 = _args[11]; -lean_object* x_13 = _args[12]; -lean_object* x_14 = _args[13]; -lean_object* x_15 = _args[14]; -lean_object* x_16 = _args[15]; -lean_object* x_17 = _args[16]; -_start: -{ -lean_object* x_18; -x_18 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +lean_object* 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_2); -lean_dec(x_1); -return x_18; -} -} -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { -_start: -{ -size_t x_14; size_t x_15; lean_object* x_16; -x_14 = lean_unbox_usize(x_4); lean_dec(x_4); -x_15 = lean_unbox_usize(x_5); -lean_dec(x_5); -x_16 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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_3); -return x_16; -} -} -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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; -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_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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_1); -return x_14; -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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) { -_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_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__8(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -return x_15; -} +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_3); +lean_ctor_set(x_24, 1, x_10); +return x_24; } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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_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_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__9(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -return x_15; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -size_t x_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_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__10(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -return x_15; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_List_allM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { -size_t x_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_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__13(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -return x_15; +lean_object* x_8; +x_8 = l_List_allM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_2); +return x_8; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___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) { _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_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__14(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -return x_15; +lean_object* x_9; +x_9 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___spec__2(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_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__15___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -size_t x_13; size_t x_14; lean_object* x_15; -x_13 = lean_unbox_usize(x_3); +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_14 = lean_unbox_usize(x_4); +x_6 = lean_unbox_usize(x_4); lean_dec(x_4); -x_15 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__15(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -return x_15; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__5___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_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_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__5___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; +x_7 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___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_Lean_Elab_withSaveInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_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) { _start: { lean_object* x_8; -x_8 = l_Lean_Elab_withSaveInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__4___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); return x_8; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, 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_7); -lean_dec(x_7); -x_17 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_16, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -lean_dec(x_4); -lean_dec(x_3); -return x_17; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: -{ -uint8_t x_17; lean_object* x_18; -x_17 = lean_unbox(x_7); -lean_dec(x_7); -x_18 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_17, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_6); -lean_dec(x_1); -return x_18; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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_7); -lean_dec(x_7); -x_18 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_17, 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_8); -return x_18; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__4___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_8); -lean_dec(x_8); -x_19 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_18, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_2); -return x_19; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_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) { _start: { -uint8_t x_16; lean_object* x_17; -x_16 = lean_unbox(x_5); -lean_dec(x_5); -x_17 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__5(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_15); +lean_object* x_12; +x_12 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_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); lean_dec(x_6); +lean_dec(x_3); lean_dec(x_2); -return x_17; +return x_12; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_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) { _start: { -size_t x_11; size_t x_12; lean_object* x_13; -x_11 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_12 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_13 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__6(x_1, x_11, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_1); +lean_object* x_13; +x_13 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_7); return x_13; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -uint8_t x_13; lean_object* x_14; -x_13 = lean_unbox(x_4); -lean_dec(x_4); -x_14 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__7(x_1, x_2, x_3, x_13, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -return x_14; +lean_object* x_12; +x_12 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_6); +return x_12; } } -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___spec__1(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -uint8_t x_5; -x_5 = lean_usize_dec_eq(x_3, x_4); -if (x_5 == 0) -{ -lean_object* x_6; lean_object* x_7; uint8_t x_8; -x_6 = lean_array_uget(x_2, x_3); -x_7 = lean_ctor_get(x_6, 1); -lean_inc(x_7); +lean_object* x_12; +x_12 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_6); -x_8 = lean_name_eq(x_7, x_1); -lean_dec(x_7); -if (x_8 == 0) -{ -size_t x_9; size_t x_10; -x_9 = 1; -x_10 = lean_usize_add(x_3, x_9); -x_3 = x_10; -goto _start; -} -else -{ -uint8_t x_12; -x_12 = 1; return x_12; } } -else -{ -uint8_t x_13; -x_13 = 0; -return x_13; -} -} -} -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___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_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___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) { _start: { -uint8_t x_9; -x_9 = lean_usize_dec_lt(x_4, x_3); -if (x_9 == 0) +uint8_t x_11; +x_11 = lean_usize_dec_lt(x_4, x_3); +if (x_11 == 0) { -lean_object* x_10; -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_5); -lean_ctor_set(x_10, 1, x_8); -return x_10; +lean_object* x_12; +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_12 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_5); +lean_ctor_set(x_12, 1, x_10); +return x_12; } else { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; -x_11 = lean_array_uget(x_2, x_4); -x_12 = lean_ctor_get(x_11, 9); -lean_inc(x_12); -x_13 = lean_array_get_size(x_12); +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_13 = lean_array_uget(x_5, x_4); x_14 = lean_unsigned_to_nat(0u); -x_15 = lean_nat_dec_lt(x_14, x_13); -if (x_15 == 0) +x_15 = lean_array_uset(x_5, x_4, x_14); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_2); +lean_inc(x_1); +x_16 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask(x_1, x_13, x_2, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_16) == 0) { -size_t x_16; size_t x_17; -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -x_16 = 1; -x_17 = lean_usize_add(x_4, x_16); -x_4 = x_17; +lean_object* x_17; lean_object* x_18; size_t x_19; size_t x_20; lean_object* x_21; +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +x_19 = 1; +x_20 = lean_usize_add(x_4, x_19); +x_21 = lean_array_uset(x_15, x_4, x_17); +x_4 = x_20; +x_5 = x_21; +x_10 = x_18; goto _start; } else { -size_t x_19; size_t x_20; uint8_t x_21; -x_19 = 0; -x_20 = lean_usize_of_nat(x_13); -lean_dec(x_13); -x_21 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___spec__1(x_1, x_12, x_19, x_20); -lean_dec(x_12); -if (x_21 == 0) +uint8_t x_23; +lean_dec(x_15); +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_23 = !lean_is_exclusive(x_16); +if (x_23 == 0) { -size_t x_22; size_t x_23; -lean_dec(x_11); -x_22 = 1; -x_23 = lean_usize_add(x_4, x_22); -x_4 = x_23; -goto _start; +return x_16; } else { -lean_object* x_25; lean_object* x_26; size_t x_27; size_t x_28; -x_25 = lean_ctor_get(x_11, 4); +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_16, 0); +x_25 = lean_ctor_get(x_16, 1); lean_inc(x_25); -lean_dec(x_11); -x_26 = lean_array_push(x_5, x_25); -x_27 = 1; -x_28 = lean_usize_add(x_4, x_27); -x_4 = x_28; -x_5 = x_26; -goto _start; +lean_inc(x_24); +lean_dec(x_16); +x_26 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_26, 0, x_24); +lean_ctor_set(x_26, 1, x_25); +return x_26; } } } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___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_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__2(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -uint8_t x_9; -x_9 = lean_usize_dec_lt(x_4, x_3); -if (x_9 == 0) +uint8_t x_10; +x_10 = lean_usize_dec_lt(x_3, x_2); +if (x_10 == 0) { -lean_object* x_10; +lean_object* x_11; +lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_5); -lean_ctor_set(x_10, 1, x_8); -return x_10; +lean_dec(x_5); +x_11 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_11, 0, x_4); +lean_ctor_set(x_11, 1, x_9); +return x_11; } else { -lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_11 = lean_array_uget(x_2, x_4); -x_12 = lean_ctor_get(x_11, 1); -lean_inc(x_12); -x_13 = l_Lean_NameSet_contains(x_5, x_12); -if (x_13 == 0) -{ -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; -x_14 = lean_box(0); -lean_inc(x_12); -x_15 = l_Lean_RBNode_insert___at_Lean_NameSet_insert___spec__1(x_5, x_12, x_14); -x_16 = lean_array_size(x_1); -x_17 = 0; -x_18 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__3___closed__1; -x_19 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___spec__2(x_12, x_1, x_16, x_17, x_18, x_6, x_7, x_8); +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_12 = lean_array_uget(x_4, x_3); +x_13 = lean_unsigned_to_nat(0u); +x_14 = lean_array_uset(x_4, x_3, x_13); +x_15 = lean_ctor_get(x_12, 1); +lean_inc(x_15); lean_dec(x_12); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_16 = l___private_Lean_Meta_Basic_0__Lean_Meta_instantiateForallAux(x_1, x_13, x_15, x_5, x_6, x_7, x_8, x_9); +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_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_19 = l_Lean_Meta_whnfD(x_17, 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; size_t x_22; size_t 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_inc(x_21); lean_dec(x_19); -lean_inc(x_7); -lean_inc(x_6); -x_22 = l_Lean_Elab_DerivingClassView_applyHandlers(x_11, x_20, x_6, x_7, x_21); -if (lean_obj_tag(x_22) == 0) -{ -lean_object* x_23; size_t x_24; size_t x_25; -x_23 = lean_ctor_get(x_22, 1); -lean_inc(x_23); -lean_dec(x_22); -x_24 = 1; -x_25 = lean_usize_add(x_4, x_24); -x_4 = x_25; -x_5 = x_15; -x_8 = x_23; +x_22 = 1; +x_23 = lean_usize_add(x_3, x_22); +x_24 = lean_array_uset(x_14, x_3, x_20); +x_3 = x_23; +x_4 = x_24; +x_9 = x_21; goto _start; } else { -uint8_t x_27; -lean_dec(x_15); +uint8_t x_26; +lean_dec(x_14); +lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -x_27 = !lean_is_exclusive(x_22); -if (x_27 == 0) +lean_dec(x_5); +x_26 = !lean_is_exclusive(x_19); +if (x_26 == 0) { -return x_22; +return x_19; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_28 = lean_ctor_get(x_22, 0); -x_29 = lean_ctor_get(x_22, 1); -lean_inc(x_29); +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_19, 0); +x_28 = lean_ctor_get(x_19, 1); lean_inc(x_28); -lean_dec(x_22); -x_30 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_30, 0, x_28); -lean_ctor_set(x_30, 1, x_29); -return x_30; +lean_inc(x_27); +lean_dec(x_19); +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_27); +lean_ctor_set(x_29, 1, x_28); +return x_29; } } } else { -size_t x_31; size_t x_32; -lean_dec(x_12); -lean_dec(x_11); -x_31 = 1; -x_32 = lean_usize_add(x_4, x_31); -x_4 = x_32; -goto _start; +uint8_t x_30; +lean_dec(x_14); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_30 = !lean_is_exclusive(x_16); +if (x_30 == 0) +{ +return x_16; +} +else +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_31 = lean_ctor_get(x_16, 0); +x_32 = lean_ctor_get(x_16, 1); +lean_inc(x_32); +lean_inc(x_31); +lean_dec(x_16); +x_33 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_33, 0, x_31); +lean_ctor_set(x_33, 1, x_32); +return x_33; } } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___spec__4(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_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___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: { -uint8_t x_9; -x_9 = lean_usize_dec_lt(x_4, x_3); -if (x_9 == 0) +if (lean_obj_tag(x_2) == 0) { -lean_object* x_10; +lean_object* x_9; lean_object* x_10; lean_dec(x_7); lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_9 = l_List_reverse___rarg(x_3); x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_5); +lean_ctor_set(x_10, 0, x_9); lean_ctor_set(x_10, 1, x_8); return x_10; } else { -lean_object* x_11; lean_object* x_12; size_t x_13; size_t x_14; lean_object* x_15; -x_11 = lean_array_uget(x_2, x_4); -x_12 = lean_ctor_get(x_11, 9); -lean_inc(x_12); -lean_dec(x_11); -x_13 = lean_array_size(x_12); -x_14 = 0; +uint8_t x_11; +x_11 = !lean_is_exclusive(x_2); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_12 = lean_ctor_get(x_2, 0); +x_13 = lean_ctor_get(x_2, 1); +x_14 = lean_ctor_get(x_12, 1); +lean_inc(x_14); +lean_dec(x_12); +x_15 = lean_unsigned_to_nat(0u); lean_inc(x_7); lean_inc(x_6); -x_15 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___spec__3(x_1, x_12, x_13, x_14, x_5, x_6, x_7, x_8); -lean_dec(x_12); -if (lean_obj_tag(x_15) == 0) +lean_inc(x_5); +lean_inc(x_4); +x_16 = l___private_Lean_Meta_Basic_0__Lean_Meta_instantiateForallAux(x_1, x_15, x_14, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_16) == 0) { -lean_object* x_16; lean_object* x_17; size_t x_18; size_t 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; +x_17 = lean_ctor_get(x_16, 0); lean_inc(x_17); -lean_dec(x_15); -x_18 = 1; -x_19 = lean_usize_add(x_4, x_18); -x_4 = x_19; -x_5 = x_16; -x_8 = x_17; +x_18 = lean_ctor_get(x_16, 1); +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_Lean_Meta_whnfD(x_17, 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; +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_19, 1); +lean_inc(x_21); +lean_dec(x_19); +lean_ctor_set(x_2, 1, x_3); +lean_ctor_set(x_2, 0, x_20); +{ +lean_object* _tmp_1 = x_13; +lean_object* _tmp_2 = x_2; +lean_object* _tmp_7 = x_21; +x_2 = _tmp_1; +x_3 = _tmp_2; +x_8 = _tmp_7; +} goto _start; } else { -uint8_t x_21; +uint8_t x_23; +lean_free_object(x_2); +lean_dec(x_13); lean_dec(x_7); lean_dec(x_6); -x_21 = !lean_is_exclusive(x_15); -if (x_21 == 0) +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_23 = !lean_is_exclusive(x_19); +if (x_23 == 0) { -return x_15; +return x_19; } else { -lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_22 = lean_ctor_get(x_15, 0); -x_23 = lean_ctor_get(x_15, 1); -lean_inc(x_23); -lean_inc(x_22); -lean_dec(x_15); -x_24 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_24, 0, x_22); -lean_ctor_set(x_24, 1, x_23); -return x_24; -} -} +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_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; } } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers(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; lean_object* x_8; -x_5 = lean_array_size(x_1); -x_6 = 0; -x_7 = l_Lean_NameSet_empty; -x_8 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___spec__4(x_1, x_1, x_5, x_6, x_7, x_2, x_3, x_4); -if (lean_obj_tag(x_8) == 0) +else { -uint8_t x_9; -x_9 = !lean_is_exclusive(x_8); -if (x_9 == 0) +uint8_t x_27; +lean_free_object(x_2); +lean_dec(x_13); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_27 = !lean_is_exclusive(x_16); +if (x_27 == 0) { -lean_object* x_10; lean_object* x_11; -x_10 = lean_ctor_get(x_8, 0); -lean_dec(x_10); -x_11 = lean_box(0); -lean_ctor_set(x_8, 0, x_11); -return x_8; +return x_16; } else { -lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_12 = lean_ctor_get(x_8, 1); -lean_inc(x_12); -lean_dec(x_8); -x_13 = lean_box(0); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_13); -lean_ctor_set(x_14, 1, x_12); -return x_14; +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_16, 0); +x_29 = lean_ctor_get(x_16, 1); +lean_inc(x_29); +lean_inc(x_28); +lean_dec(x_16); +x_30 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +return x_30; +} } } else { -uint8_t x_15; -x_15 = !lean_is_exclusive(x_8); -if (x_15 == 0) +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_31 = lean_ctor_get(x_2, 0); +x_32 = lean_ctor_get(x_2, 1); +lean_inc(x_32); +lean_inc(x_31); +lean_dec(x_2); +x_33 = lean_ctor_get(x_31, 1); +lean_inc(x_33); +lean_dec(x_31); +x_34 = lean_unsigned_to_nat(0u); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_35 = l___private_Lean_Meta_Basic_0__Lean_Meta_instantiateForallAux(x_1, x_34, x_33, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_35) == 0) { -return x_8; +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_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_38 = l_Lean_Meta_whnfD(x_36, x_4, x_5, x_6, x_7, x_37); +if (lean_obj_tag(x_38) == 0) +{ +lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = lean_ctor_get(x_38, 0); +lean_inc(x_39); +x_40 = lean_ctor_get(x_38, 1); +lean_inc(x_40); +lean_dec(x_38); +x_41 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_41, 0, x_39); +lean_ctor_set(x_41, 1, x_3); +x_2 = x_32; +x_3 = x_41; +x_8 = x_40; +goto _start; } else { -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_8, 0); -x_17 = lean_ctor_get(x_8, 1); -lean_inc(x_17); -lean_inc(x_16); -lean_dec(x_8); -x_18 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_18, 0, x_16); -lean_ctor_set(x_18, 1, x_17); -return x_18; +lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; +lean_dec(x_32); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_43 = lean_ctor_get(x_38, 0); +lean_inc(x_43); +x_44 = lean_ctor_get(x_38, 1); +lean_inc(x_44); +if (lean_is_exclusive(x_38)) { + lean_ctor_release(x_38, 0); + lean_ctor_release(x_38, 1); + x_45 = x_38; +} else { + lean_dec_ref(x_38); + x_45 = lean_box(0); } +if (lean_is_scalar(x_45)) { + x_46 = lean_alloc_ctor(1, 2, 0); +} else { + x_46 = x_45; } +lean_ctor_set(x_46, 0, x_43); +lean_ctor_set(x_46, 1, x_44); +return x_46; } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___spec__1___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_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +lean_dec(x_32); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); -x_7 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___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_dec(x_3); +x_47 = lean_ctor_get(x_35, 0); +lean_inc(x_47); +x_48 = lean_ctor_get(x_35, 1); +lean_inc(x_48); +if (lean_is_exclusive(x_35)) { + lean_ctor_release(x_35, 0); + lean_ctor_release(x_35, 1); + x_49 = x_35; +} else { + lean_dec_ref(x_35); + x_49 = lean_box(0); } +if (lean_is_scalar(x_49)) { + x_50 = lean_alloc_ctor(1, 2, 0); +} else { + x_50 = x_49; } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___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) { -_start: -{ -size_t x_9; size_t x_10; lean_object* x_11; -x_9 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_10 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_11 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___spec__2(x_1, x_2, x_9, x_10, x_5, x_6, x_7, x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_2); -lean_dec(x_1); -return x_11; +lean_ctor_set(x_50, 0, x_47); +lean_ctor_set(x_50, 1, x_48); +return x_50; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___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: -{ -size_t x_9; size_t x_10; lean_object* x_11; -x_9 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_10 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_11 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___spec__3(x_1, x_2, x_9, x_10, x_5, x_6, x_7, x_8); -lean_dec(x_2); -lean_dec(x_1); -return x_11; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___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_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -size_t x_9; size_t x_10; lean_object* x_11; -x_9 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_10 = lean_unbox_usize(x_4); +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_9; lean_object* x_10; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); -x_11 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___spec__4(x_1, x_2, x_9, x_10, x_5, x_6, x_7, x_8); -lean_dec(x_2); -lean_dec(x_1); -return x_11; -} +x_9 = l_List_reverse___rarg(x_3); +x_10 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set(x_10, 1, x_8); +return x_10; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers(x_1, x_2, x_3, x_4); -lean_dec(x_1); -return x_5; -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__1() { -_start: +uint8_t x_11; +x_11 = !lean_is_exclusive(x_2); +if (x_11 == 0) { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Parser", 6, 6); -return x_1; -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__2() { -_start: +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); +x_13 = lean_ctor_get(x_2, 1); +x_14 = lean_ctor_get(x_12, 2); +lean_inc(x_14); +lean_dec(x_12); +x_15 = lean_box(0); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_16 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__3(x_1, x_14, x_15, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_16) == 0) { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("declaration", 11, 11); -return x_1; -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__3() { -_start: +lean_object* x_17; lean_object* x_18; +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_2, 1, x_3); +lean_ctor_set(x_2, 0, x_17); { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__1; -x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__7; -x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__2; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; +lean_object* _tmp_1 = x_13; +lean_object* _tmp_2 = x_2; +lean_object* _tmp_7 = x_18; +x_2 = _tmp_1; +x_3 = _tmp_2; +x_8 = _tmp_7; } +goto _start; } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__4() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("definition", 10, 10); -return x_1; -} +uint8_t x_20; +lean_free_object(x_2); +lean_dec(x_13); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_20 = !lean_is_exclusive(x_16); +if (x_20 == 0) +{ +return x_16; } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__5() { -_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_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__1; -x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__7; -x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__4; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; +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; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__6() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("def", 3, 3); -return x_1; } +else +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_24 = lean_ctor_get(x_2, 0); +x_25 = lean_ctor_get(x_2, 1); +lean_inc(x_25); +lean_inc(x_24); +lean_dec(x_2); +x_26 = lean_ctor_get(x_24, 2); +lean_inc(x_26); +lean_dec(x_24); +x_27 = lean_box(0); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_28 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__3(x_1, x_26, x_27, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_28) == 0) +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_28, 0); +lean_inc(x_29); +x_30 = lean_ctor_get(x_28, 1); +lean_inc(x_30); +lean_dec(x_28); +x_31 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_31, 0, x_29); +lean_ctor_set(x_31, 1, x_3); +x_2 = x_25; +x_3 = x_31; +x_8 = x_30; +goto _start; } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__7() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("declId", 6, 6); -return x_1; +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; +lean_dec(x_25); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_33 = lean_ctor_get(x_28, 0); +lean_inc(x_33); +x_34 = lean_ctor_get(x_28, 1); +lean_inc(x_34); +if (lean_is_exclusive(x_28)) { + lean_ctor_release(x_28, 0); + lean_ctor_release(x_28, 1); + x_35 = x_28; +} else { + lean_dec_ref(x_28); + x_35 = lean_box(0); +} +if (lean_is_scalar(x_35)) { + x_36 = lean_alloc_ctor(1, 2, 0); +} else { + x_36 = x_35; +} +lean_ctor_set(x_36, 0, x_33); +lean_ctor_set(x_36, 1, x_34); +return x_36; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__8() { +} +} +} +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__5(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__1; -x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__7; -x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__7; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_3; +x_3 = lean_array_to_list(x_2); +return x_3; } +else +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +x_5 = lean_ctor_get(x_1, 1); +lean_inc(x_5); +lean_dec(x_1); +x_6 = l_List_foldl___at_Array_appendList___spec__1___rarg(x_2, x_4); +x_1 = x_5; +x_2 = x_6; +goto _start; } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__9() { +} +} +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__7(uint8_t x_1, lean_object* x_2, size_t x_3, size_t x_4) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("_root_", 6, 6); -return x_1; +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_unbox(x_6); +lean_dec(x_6); +if (x_7 == 0) +{ +if (x_1 == 0) +{ +uint8_t x_8; +x_8 = 1; +return x_8; +} +else +{ +size_t x_9; size_t x_10; +x_9 = 1; +x_10 = lean_usize_add(x_3, x_9); +x_3 = x_10; +goto _start; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__10() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__9; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +if (x_1 == 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; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__11() { -_start: +} +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("null", 4, 4); -return x_1; +uint8_t x_16; +x_16 = 0; +return x_16; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__12() { +} +LEAN_EXPORT uint8_t l_Array_contains___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__6(lean_object* x_1, uint8_t x_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_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__11; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +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 +{ +size_t x_7; size_t x_8; uint8_t x_9; +x_7 = 0; +x_8 = lean_usize_of_nat(x_3); +lean_dec(x_3); +x_9 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__7(x_2, x_1, x_7, x_8); +return x_9; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__13() { +} +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__8(lean_object* x_1, size_t x_2, size_t x_3) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("optDeclSig", 10, 10); -return x_1; +uint8_t x_4; +x_4 = lean_usize_dec_eq(x_2, x_3); +if (x_4 == 0) +{ +lean_object* x_5; uint8_t x_6; uint8_t x_7; +x_5 = lean_array_uget(x_1, x_2); +x_6 = 1; +x_7 = l_Array_contains___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__6(x_5, x_6); +lean_dec(x_5); +if (x_7 == 0) +{ +size_t x_8; size_t x_9; +x_8 = 1; +x_9 = lean_usize_add(x_2, x_8); +x_2 = x_9; +goto _start; +} +else +{ +uint8_t x_11; +x_11 = 1; +return x_11; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__14() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__1; -x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__7; -x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__13; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; +uint8_t x_12; +x_12 = 0; +return x_12; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__15() { +} +LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Term", 4, 4); -return x_1; +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; lean_object* x_8; lean_object* x_9; +x_6 = lean_ctor_get(x_2, 0); +x_7 = lean_ctor_get(x_2, 1); +lean_inc(x_1); +x_8 = lean_apply_1(x_1, x_6); +x_9 = l_Lean_MessageData_ofFormat(x_8); +lean_ctor_set(x_2, 1, x_3); +lean_ctor_set(x_2, 0, x_9); +{ +lean_object* _tmp_1 = x_7; +lean_object* _tmp_2 = x_2; +x_2 = _tmp_1; +x_3 = _tmp_2; } +goto _start; } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__16() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("typeSpec", 8, 8); -return x_1; +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_11 = lean_ctor_get(x_2, 0); +x_12 = lean_ctor_get(x_2, 1); +lean_inc(x_12); +lean_inc(x_11); +lean_dec(x_2); +lean_inc(x_1); +x_13 = lean_apply_1(x_1, x_11); +x_14 = l_Lean_MessageData_ofFormat(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_3); +x_2 = x_12; +x_3 = x_15; +goto _start; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__17() { +} +} +LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__1; -x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__15; -x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__16; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +if (lean_obj_tag(x_3) == 0) +{ +lean_object* x_5; +lean_dec(x_2); +lean_dec(x_1); +x_5 = l_List_reverse___rarg(x_4); return x_5; } +else +{ +uint8_t x_6; +x_6 = !lean_is_exclusive(x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_7 = lean_ctor_get(x_3, 0); +x_8 = lean_ctor_get(x_3, 1); +lean_inc(x_2); +x_9 = lean_apply_1(x_2, x_7); +lean_inc(x_1); +x_10 = lean_apply_1(x_1, x_9); +x_11 = l_Lean_MessageData_ofFormat(x_10); +lean_ctor_set(x_3, 1, x_4); +lean_ctor_set(x_3, 0, x_11); +{ +lean_object* _tmp_2 = x_8; +lean_object* _tmp_3 = x_3; +x_3 = _tmp_2; +x_4 = _tmp_3; +} +goto _start; } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__18() { +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; +x_13 = lean_ctor_get(x_3, 0); +x_14 = lean_ctor_get(x_3, 1); +lean_inc(x_14); +lean_inc(x_13); +lean_dec(x_3); +lean_inc(x_2); +x_15 = lean_apply_1(x_2, x_13); +lean_inc(x_1); +x_16 = lean_apply_1(x_1, x_15); +x_17 = l_Lean_MessageData_ofFormat(x_16); +x_18 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set(x_18, 1, x_4); +x_3 = x_14; +x_4 = x_18; +goto _start; +} +} +} +} +static lean_object* _init_l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked(":", 1, 1); +x_1 = lean_mk_string_unchecked("false", 5, 5); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__19() { +static lean_object* _init_l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("declValEqns", 11, 11); -return x_1; +lean_object* x_1; lean_object* x_2; +x_1 = l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11___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_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__20() { +static lean_object* _init_l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11___closed__3() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__1; -x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__7; -x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__19; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; +lean_object* x_1; lean_object* x_2; +x_1 = l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11___closed__2; +x_2 = l_Lean_MessageData_ofFormat(x_1); +return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__21() { +static lean_object* _init_l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11___closed__4() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("matchAltsWhereDecls", 19, 19); +x_1 = lean_mk_string_unchecked("true", 4, 4); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__22() { +static lean_object* _init_l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11___closed__5() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__1; -x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__15; -x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__21; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; +lean_object* x_1; lean_object* x_2; +x_1 = l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11___closed__4; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__23() { +static lean_object* _init_l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11___closed__6() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Termination", 11, 11); -return x_1; +lean_object* x_1; lean_object* x_2; +x_1 = l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11___closed__5; +x_2 = l_Lean_MessageData_ofFormat(x_1); +return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__24() { +LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("suffix", 6, 6); -return x_1; +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_3; +x_3 = l_List_reverse___rarg(x_2); +return x_3; } +else +{ +lean_object* x_4; uint8_t x_5; +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +x_5 = lean_unbox(x_4); +lean_dec(x_4); +if (x_5 == 0) +{ +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; +x_7 = lean_ctor_get(x_1, 1); +x_8 = lean_ctor_get(x_1, 0); +lean_dec(x_8); +x_9 = l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11___closed__3; +lean_ctor_set(x_1, 1, x_2); +lean_ctor_set(x_1, 0, x_9); +{ +lean_object* _tmp_0 = x_7; +lean_object* _tmp_1 = x_1; +x_1 = _tmp_0; +x_2 = _tmp_1; } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__25() { -_start: +goto _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_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__1; -x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__23; -x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__24; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_1, 1); +lean_inc(x_11); +lean_dec(x_1); +x_12 = l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11___closed__3; +x_13 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_2); +x_1 = x_11; +x_2 = x_13; +goto _start; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +else { -lean_object* x_10; uint8_t x_11; -x_10 = l_Lean_Elab_Command_getRef(x_7, x_8, x_9); -x_11 = !lean_is_exclusive(x_10); -if (x_11 == 0) +uint8_t x_15; +x_15 = !lean_is_exclusive(x_1); +if (x_15 == 0) { -lean_object* x_12; lean_object* x_13; uint8_t x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; -x_12 = lean_ctor_get(x_10, 0); -x_13 = lean_ctor_get(x_10, 1); -x_14 = 0; -x_15 = l_Lean_SourceInfo_fromRef(x_12, x_14); -lean_dec(x_12); -x_16 = l_Lean_Elab_Command_getCurrMacroScope(x_7, x_8, x_13); -x_17 = !lean_is_exclusive(x_16); -if (x_17 == 0) +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_1, 1); +x_17 = lean_ctor_get(x_1, 0); +lean_dec(x_17); +x_18 = l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11___closed__6; +lean_ctor_set(x_1, 1, x_2); +lean_ctor_set(x_1, 0, x_18); { -lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; -x_18 = lean_ctor_get(x_16, 1); -x_19 = lean_ctor_get(x_16, 0); -lean_dec(x_19); -x_20 = l_Lean_Elab_Command_getMainModule___rarg(x_8, x_18); -x_21 = !lean_is_exclusive(x_20); -if (x_21 == 0) +lean_object* _tmp_0 = x_16; +lean_object* _tmp_1 = x_1; +x_1 = _tmp_0; +x_2 = _tmp_1; +} +goto _start; +} +else { -lean_object* x_22; uint8_t x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_22 = lean_ctor_get(x_20, 0); -lean_dec(x_22); -x_23 = 1; -x_24 = l_Lean_SourceInfo_fromRef(x_1, x_23); -x_25 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__6; -lean_ctor_set_tag(x_16, 2); -lean_ctor_set(x_16, 1, x_25); -lean_ctor_set(x_16, 0, x_24); -x_26 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__10; -x_27 = l_Lean_Name_append(x_26, x_2); -x_28 = l_Lean_Name_append(x_27, x_3); -x_29 = lean_mk_syntax_ident(x_28); -x_30 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__12; -x_31 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; -lean_inc(x_15); -x_32 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_32, 0, x_15); -lean_ctor_set(x_32, 1, x_30); -lean_ctor_set(x_32, 2, x_31); -x_33 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__8; -lean_inc(x_32); -lean_inc(x_15); -x_34 = l_Lean_Syntax_node2(x_15, x_33, x_29, x_32); -x_35 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__18; -lean_inc(x_15); -lean_ctor_set_tag(x_10, 2); -lean_ctor_set(x_10, 1, x_35); -lean_ctor_set(x_10, 0, x_15); -x_36 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__17; -lean_inc(x_15); -x_37 = l_Lean_Syntax_node2(x_15, x_36, x_10, x_4); -lean_inc(x_15); -x_38 = l_Lean_Syntax_node1(x_15, x_30, x_37); -x_39 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__14; -lean_inc(x_32); -lean_inc(x_15); -x_40 = l_Lean_Syntax_node2(x_15, x_39, x_32, x_38); -x_41 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__25; -lean_inc_n(x_32, 2); -lean_inc(x_15); -x_42 = l_Lean_Syntax_node2(x_15, x_41, x_32, x_32); -x_43 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__22; -lean_inc(x_32); -lean_inc(x_15); -x_44 = l_Lean_Syntax_node3(x_15, x_43, x_5, x_42, x_32); -x_45 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__20; -lean_inc(x_15); -x_46 = l_Lean_Syntax_node1(x_15, x_45, x_44); -x_47 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__5; -lean_inc(x_15); -x_48 = l_Lean_Syntax_node5(x_15, x_47, x_16, x_34, x_40, x_46, x_32); -x_49 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__3; -x_50 = l_Lean_Syntax_node2(x_15, x_49, x_6, x_48); -lean_ctor_set(x_20, 0, x_50); -return x_20; +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_1, 1); +lean_inc(x_20); +lean_dec(x_1); +x_21 = l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11___closed__6; +x_22 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_22, 0, x_21); +lean_ctor_set(x_22, 1, x_2); +x_1 = x_20; +x_2 = x_22; +goto _start; +} +} +} +} +} +LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__12(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 { -lean_object* x_51; uint8_t x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; -x_51 = lean_ctor_get(x_20, 1); -lean_inc(x_51); -lean_dec(x_20); -x_52 = 1; -x_53 = l_Lean_SourceInfo_fromRef(x_1, x_52); -x_54 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__6; -lean_ctor_set_tag(x_16, 2); -lean_ctor_set(x_16, 1, x_54); -lean_ctor_set(x_16, 0, x_53); -x_55 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__10; -x_56 = l_Lean_Name_append(x_55, x_2); -x_57 = l_Lean_Name_append(x_56, x_3); -x_58 = lean_mk_syntax_ident(x_57); -x_59 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__12; -x_60 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; -lean_inc(x_15); -x_61 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_61, 0, x_15); -lean_ctor_set(x_61, 1, x_59); -lean_ctor_set(x_61, 2, x_60); -x_62 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__8; -lean_inc(x_61); -lean_inc(x_15); -x_63 = l_Lean_Syntax_node2(x_15, x_62, x_58, x_61); -x_64 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__18; -lean_inc(x_15); -lean_ctor_set_tag(x_10, 2); -lean_ctor_set(x_10, 1, x_64); -lean_ctor_set(x_10, 0, x_15); -x_65 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__17; -lean_inc(x_15); -x_66 = l_Lean_Syntax_node2(x_15, x_65, x_10, x_4); -lean_inc(x_15); -x_67 = l_Lean_Syntax_node1(x_15, x_59, x_66); -x_68 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__14; -lean_inc(x_61); -lean_inc(x_15); -x_69 = l_Lean_Syntax_node2(x_15, x_68, x_61, x_67); -x_70 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__25; -lean_inc_n(x_61, 2); -lean_inc(x_15); -x_71 = l_Lean_Syntax_node2(x_15, x_70, x_61, x_61); -x_72 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__22; -lean_inc(x_61); -lean_inc(x_15); -x_73 = l_Lean_Syntax_node3(x_15, x_72, x_5, x_71, x_61); -x_74 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__20; -lean_inc(x_15); -x_75 = l_Lean_Syntax_node1(x_15, x_74, x_73); -x_76 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__5; -lean_inc(x_15); -x_77 = l_Lean_Syntax_node5(x_15, x_76, x_16, x_63, x_69, x_75, x_61); -x_78 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__3; -x_79 = l_Lean_Syntax_node2(x_15, x_78, x_6, x_77); -x_80 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_80, 0, x_79); -lean_ctor_set(x_80, 1, x_51); -return x_80; +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; lean_object* x_10; +x_5 = lean_ctor_get(x_1, 0); +x_6 = lean_ctor_get(x_1, 1); +x_7 = lean_array_to_list(x_5); +x_8 = lean_box(0); +x_9 = l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11(x_7, x_8); +x_10 = l_Lean_MessageData_ofList(x_9); +lean_ctor_set(x_1, 1, x_2); +lean_ctor_set(x_1, 0, x_10); +{ +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_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; uint8_t x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; -x_81 = lean_ctor_get(x_16, 1); -lean_inc(x_81); -lean_dec(x_16); -x_82 = l_Lean_Elab_Command_getMainModule___rarg(x_8, x_81); -x_83 = lean_ctor_get(x_82, 1); -lean_inc(x_83); -if (lean_is_exclusive(x_82)) { - lean_ctor_release(x_82, 0); - lean_ctor_release(x_82, 1); - x_84 = x_82; -} else { - lean_dec_ref(x_82); - x_84 = lean_box(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; +x_12 = lean_ctor_get(x_1, 0); +x_13 = lean_ctor_get(x_1, 1); +lean_inc(x_13); +lean_inc(x_12); +lean_dec(x_1); +x_14 = lean_array_to_list(x_12); +x_15 = lean_box(0); +x_16 = l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__10___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__11(x_14, x_15); +x_17 = l_Lean_MessageData_ofList(x_16); +x_18 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set(x_18, 1, x_2); +x_1 = x_13; +x_2 = x_18; +goto _start; } -x_85 = 1; -x_86 = l_Lean_SourceInfo_fromRef(x_1, x_85); -x_87 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__6; -x_88 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_88, 0, x_86); -lean_ctor_set(x_88, 1, x_87); -x_89 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__10; -x_90 = l_Lean_Name_append(x_89, x_2); -x_91 = l_Lean_Name_append(x_90, x_3); -x_92 = lean_mk_syntax_ident(x_91); -x_93 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__12; -x_94 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; -lean_inc(x_15); -x_95 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_95, 0, x_15); -lean_ctor_set(x_95, 1, x_93); -lean_ctor_set(x_95, 2, x_94); -x_96 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__8; -lean_inc(x_95); -lean_inc(x_15); -x_97 = l_Lean_Syntax_node2(x_15, x_96, x_92, x_95); -x_98 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__18; -lean_inc(x_15); -lean_ctor_set_tag(x_10, 2); -lean_ctor_set(x_10, 1, x_98); -lean_ctor_set(x_10, 0, x_15); -x_99 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__17; -lean_inc(x_15); -x_100 = l_Lean_Syntax_node2(x_15, x_99, x_10, x_4); -lean_inc(x_15); -x_101 = l_Lean_Syntax_node1(x_15, x_93, x_100); -x_102 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__14; -lean_inc(x_95); -lean_inc(x_15); -x_103 = l_Lean_Syntax_node2(x_15, x_102, x_95, x_101); -x_104 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__25; -lean_inc_n(x_95, 2); -lean_inc(x_15); -x_105 = l_Lean_Syntax_node2(x_15, x_104, x_95, x_95); -x_106 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__22; -lean_inc(x_95); -lean_inc(x_15); -x_107 = l_Lean_Syntax_node3(x_15, x_106, x_5, x_105, x_95); -x_108 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__20; -lean_inc(x_15); -x_109 = l_Lean_Syntax_node1(x_15, x_108, x_107); -x_110 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__5; -lean_inc(x_15); -x_111 = l_Lean_Syntax_node5(x_15, x_110, x_88, x_97, x_103, x_109, x_95); -x_112 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__3; -x_113 = l_Lean_Syntax_node2(x_15, x_112, x_6, x_111); -if (lean_is_scalar(x_84)) { - x_114 = lean_alloc_ctor(0, 2, 0); -} else { - x_114 = x_84; } -lean_ctor_set(x_114, 0, x_113); -lean_ctor_set(x_114, 1, x_83); -return x_114; } } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__1(lean_object* x_1, size_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; size_t x_17; lean_object* x_18; +x_13 = lean_array_get_size(x_1); +x_14 = lean_unsigned_to_nat(1u); +lean_inc(x_1); +x_15 = l_Array_toSubarray___rarg(x_1, x_14, x_13); +x_16 = l_Array_ofSubarray___rarg(x_15); +lean_dec(x_15); +x_17 = lean_array_size(x_16); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +x_18 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__2(x_6, x_17, x_2, x_16, x_8, x_9, x_10, x_11, x_12); +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; +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +x_20 = lean_ctor_get(x_18, 1); +lean_inc(x_20); +lean_dec(x_18); +x_21 = lean_array_to_list(x_1); +x_22 = lean_box(0); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +x_23 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__4(x_6, x_21, x_22, x_8, x_9, x_10, x_11, x_20); +if (lean_obj_tag(x_23) == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +x_26 = lean_array_to_list(x_19); +x_27 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__8___closed__1; +x_28 = l_List_flatMapTR_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__5(x_24, x_27); +x_29 = l_List_appendTR___rarg(x_26, x_28); +x_30 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go(x_3, x_4, x_5, x_7, x_29, x_8, x_9, x_10, x_11, x_25); +return x_30; +} else { -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; uint8_t x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; -x_115 = lean_ctor_get(x_10, 0); -x_116 = lean_ctor_get(x_10, 1); -lean_inc(x_116); -lean_inc(x_115); +uint8_t x_31; +lean_dec(x_19); +lean_dec(x_11); lean_dec(x_10); -x_117 = 0; -x_118 = l_Lean_SourceInfo_fromRef(x_115, x_117); -lean_dec(x_115); -x_119 = l_Lean_Elab_Command_getCurrMacroScope(x_7, x_8, x_116); -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); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_31 = !lean_is_exclusive(x_23); +if (x_31 == 0) +{ +return x_23; } -x_122 = l_Lean_Elab_Command_getMainModule___rarg(x_8, 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_122); - x_124 = lean_box(0); +else +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_23, 0); +x_33 = lean_ctor_get(x_23, 1); +lean_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; } -x_125 = 1; -x_126 = l_Lean_SourceInfo_fromRef(x_1, x_125); -x_127 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__6; -if (lean_is_scalar(x_121)) { - x_128 = lean_alloc_ctor(2, 2, 0); -} else { - x_128 = x_121; - lean_ctor_set_tag(x_128, 2); } -lean_ctor_set(x_128, 0, x_126); -lean_ctor_set(x_128, 1, x_127); -x_129 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__10; -x_130 = l_Lean_Name_append(x_129, x_2); -x_131 = l_Lean_Name_append(x_130, x_3); -x_132 = lean_mk_syntax_ident(x_131); -x_133 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__12; -x_134 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; -lean_inc(x_118); -x_135 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_135, 0, x_118); -lean_ctor_set(x_135, 1, x_133); -lean_ctor_set(x_135, 2, x_134); -x_136 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__8; -lean_inc(x_135); -lean_inc(x_118); -x_137 = l_Lean_Syntax_node2(x_118, x_136, x_132, x_135); -x_138 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__18; -lean_inc(x_118); -x_139 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_139, 0, x_118); -lean_ctor_set(x_139, 1, x_138); -x_140 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__17; -lean_inc(x_118); -x_141 = l_Lean_Syntax_node2(x_118, x_140, x_139, x_4); -lean_inc(x_118); -x_142 = l_Lean_Syntax_node1(x_118, x_133, x_141); -x_143 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__14; -lean_inc(x_135); -lean_inc(x_118); -x_144 = l_Lean_Syntax_node2(x_118, x_143, x_135, x_142); -x_145 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__25; -lean_inc_n(x_135, 2); -lean_inc(x_118); -x_146 = l_Lean_Syntax_node2(x_118, x_145, x_135, x_135); -x_147 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__22; -lean_inc(x_135); -lean_inc(x_118); -x_148 = l_Lean_Syntax_node3(x_118, x_147, x_5, x_146, x_135); -x_149 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__20; -lean_inc(x_118); -x_150 = l_Lean_Syntax_node1(x_118, x_149, x_148); -x_151 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__5; -lean_inc(x_118); -x_152 = l_Lean_Syntax_node5(x_118, x_151, x_128, x_137, x_144, x_150, x_135); -x_153 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__3; -x_154 = l_Lean_Syntax_node2(x_118, x_153, x_6, x_152); -if (lean_is_scalar(x_124)) { - x_155 = lean_alloc_ctor(0, 2, 0); -} else { - x_155 = x_124; } -lean_ctor_set(x_155, 0, x_154); -lean_ctor_set(x_155, 1, x_123); -return x_155; +else +{ +uint8_t x_35; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_35 = !lean_is_exclusive(x_18); +if (x_35 == 0) +{ +return x_18; +} +else +{ +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_18, 0); +x_37 = lean_ctor_get(x_18, 1); +lean_inc(x_37); +lean_inc(x_36); +lean_dec(x_18); +x_38 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_38, 0, x_36); +lean_ctor_set(x_38, 1, x_37); +return x_38; } } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__1() { +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("unsupported modifiers for computed field", 40, 40); -return x_1; +lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; uint8_t x_15; lean_object* x_16; lean_object* x_17; +x_11 = lean_array_get_size(x_1); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_nat_dec_lt(x_12, x_11); +lean_dec(x_11); +x_14 = lean_array_get_size(x_2); +x_15 = lean_nat_dec_lt(x_12, x_14); +lean_dec(x_14); +lean_inc(x_3); +x_16 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_16, 0, x_3); +if (x_13 == 0) +{ +lean_object* x_30; lean_object* x_31; +x_30 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; +x_31 = l_outOfBounds___rarg(x_30); +x_17 = x_31; +goto block_29; } +else +{ +lean_object* x_32; +x_32 = lean_array_fget(x_1, x_12); +x_17 = x_32; +goto block_29; } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__2() { -_start: +block_29: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__1; -x_2 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; +lean_object* x_18; lean_object* x_19; +x_18 = lean_box_usize(x_4); +lean_inc(x_2); +x_19 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__1___boxed), 12, 5); +lean_closure_set(x_19, 0, x_2); +lean_closure_set(x_19, 1, x_18); +lean_closure_set(x_19, 2, x_1); +lean_closure_set(x_19, 3, x_17); +lean_closure_set(x_19, 4, x_3); +if (x_15 == 0) +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; lean_object* x_24; +lean_dec(x_2); +x_20 = l_Lean_instInhabitedInductiveType; +x_21 = l_outOfBounds___rarg(x_20); +x_22 = lean_ctor_get(x_21, 1); +lean_inc(x_22); +lean_dec(x_21); +x_23 = 0; +x_24 = l_Lean_Meta_forallBoundedTelescope___at_Lean_Meta_arrowDomainsN___spec__6___rarg(x_22, x_16, x_19, x_23, x_6, x_7, x_8, x_9, x_10); +return x_24; +} +else +{ +lean_object* x_25; lean_object* x_26; uint8_t x_27; lean_object* x_28; +x_25 = lean_array_fget(x_2, x_12); +lean_dec(x_2); +x_26 = lean_ctor_get(x_25, 1); +lean_inc(x_26); +lean_dec(x_25); +x_27 = 0; +x_28 = l_Lean_Meta_forallBoundedTelescope___at_Lean_Meta_arrowDomainsN___spec__6___rarg(x_26, x_16, x_19, x_27, x_6, x_7, x_8, x_9, x_10); +return x_28; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__3() { +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__2; -x_2 = l_Lean_MessageData_ofFormat(x_1); -return x_2; +lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_11 = lean_array_get_size(x_1); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_nat_dec_lt(x_12, x_11); +if (x_13 == 0) +{ +lean_object* x_14; +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_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_3); +lean_ctor_set(x_14, 1, x_10); +return x_14; +} +else +{ +size_t x_15; uint8_t x_16; +x_15 = lean_usize_of_nat(x_11); +lean_dec(x_11); +x_16 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__8(x_1, x_4, x_15); +if (x_16 == 0) +{ +lean_object* x_17; +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_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_3); +lean_ctor_set(x_17, 1, x_10); +return x_17; } +else +{ +lean_object* x_18; lean_object* x_19; +x_18 = lean_box(0); +x_19 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__2(x_1, x_2, x_3, x_4, x_18, x_6, x_7, x_8, x_9, x_10); +return x_19; } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4() { +} +} +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__4___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("noncomputable", 13, 13); +x_1 = lean_mk_string_unchecked("masks: ", 7, 7); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__1; -x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__7; -x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__6() { +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__4___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; -x_2 = l_Array_append___rarg(x_1, x_1); +x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__4___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; -x_11 = lean_unsigned_to_nat(4u); -x_12 = l_Lean_Syntax_getArg(x_1, x_11); -x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Syntax_matchesNull(x_12, x_13); -if (x_14 == 0) +size_t x_10; size_t x_11; lean_object* x_12; +x_10 = lean_array_size(x_1); +x_11 = 0; +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_1); +lean_inc(x_2); +x_12 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__1(x_2, x_3, x_10, x_11, x_1, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_12) == 0) { -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t 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; uint8_t x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -x_15 = l_Lean_Elab_Command_getRef(x_8, x_9, x_10); -x_16 = lean_ctor_get(x_15, 0); -lean_inc(x_16); -x_17 = lean_ctor_get(x_15, 1); +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_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_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__3; +x_16 = l_Lean_isTracingEnabledFor___at_Lean_Meta_processPostponed_loop___spec__1(x_15, x_5, x_6, x_7, x_8, x_14); +x_17 = lean_ctor_get(x_16, 0); lean_inc(x_17); -lean_dec(x_15); -x_18 = l_Lean_replaceRef(x_1, x_16); -lean_dec(x_16); -x_19 = lean_ctor_get(x_8, 0); +x_18 = lean_unbox(x_17); +lean_dec(x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_16, 1); lean_inc(x_19); -x_20 = lean_ctor_get(x_8, 1); -lean_inc(x_20); -x_21 = lean_ctor_get(x_8, 2); -lean_inc(x_21); -x_22 = lean_ctor_get(x_8, 3); -lean_inc(x_22); -x_23 = lean_ctor_get(x_8, 4); -lean_inc(x_23); -x_24 = lean_ctor_get(x_8, 5); -lean_inc(x_24); -x_25 = lean_ctor_get(x_8, 7); -lean_inc(x_25); -x_26 = lean_ctor_get(x_8, 8); -lean_inc(x_26); -x_27 = lean_ctor_get(x_8, 9); -lean_inc(x_27); -x_28 = lean_ctor_get_uint8(x_8, sizeof(void*)*10); -x_29 = lean_alloc_ctor(0, 10, 1); -lean_ctor_set(x_29, 0, x_19); -lean_ctor_set(x_29, 1, x_20); -lean_ctor_set(x_29, 2, x_21); -lean_ctor_set(x_29, 3, x_22); -lean_ctor_set(x_29, 4, x_23); -lean_ctor_set(x_29, 5, x_24); -lean_ctor_set(x_29, 6, x_18); -lean_ctor_set(x_29, 7, x_25); -lean_ctor_set(x_29, 8, x_26); -lean_ctor_set(x_29, 9, x_27); -lean_ctor_set_uint8(x_29, sizeof(void*)*10, 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; -x_32 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_30, x_31, x_29, x_9, x_17); -x_33 = lean_ctor_get(x_32, 1); +lean_dec(x_16); +x_20 = lean_box(0); +x_21 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__3(x_13, x_1, x_2, x_11, x_20, x_5, x_6, x_7, x_8, x_19); +return x_21; +} +else +{ +uint8_t x_22; +x_22 = !lean_is_exclusive(x_16); +if (x_22 == 0) +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_23 = lean_ctor_get(x_16, 1); +x_24 = lean_ctor_get(x_16, 0); +lean_dec(x_24); +lean_inc(x_13); +x_25 = lean_array_to_list(x_13); +x_26 = lean_box(0); +x_27 = l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__12(x_25, x_26); +x_28 = l_Lean_MessageData_ofList(x_27); +x_29 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__4___closed__2; +lean_ctor_set_tag(x_16, 7); +lean_ctor_set(x_16, 1, x_28); +lean_ctor_set(x_16, 0, x_29); +x_30 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +x_31 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_31, 0, x_16); +lean_ctor_set(x_31, 1, x_30); +x_32 = l_Lean_addTrace___at_Lean_Meta_processPostponed_loop___spec__2(x_15, x_31, x_5, x_6, x_7, x_8, x_23); +x_33 = lean_ctor_get(x_32, 0); lean_inc(x_33); +x_34 = lean_ctor_get(x_32, 1); +lean_inc(x_34); lean_dec(x_32); -x_34 = l_Lean_Elab_Command_getRef(x_8, x_9, x_33); -x_35 = lean_ctor_get(x_34, 0); -lean_inc(x_35); -x_36 = lean_ctor_get(x_34, 1); -lean_inc(x_36); -lean_dec(x_34); -x_37 = 0; -x_38 = l_Lean_SourceInfo_fromRef(x_35, x_37); -lean_dec(x_35); -x_39 = l_Lean_Elab_Command_getCurrMacroScope(x_8, x_9, x_36); -x_40 = lean_ctor_get(x_39, 1); -lean_inc(x_40); -lean_dec(x_39); -x_41 = l_Lean_Elab_Command_getMainModule___rarg(x_9, x_40); -x_42 = !lean_is_exclusive(x_41); -if (x_42 == 0) -{ -lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; -x_43 = lean_ctor_get(x_41, 1); -x_44 = lean_ctor_get(x_41, 0); -lean_dec(x_44); -x_45 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__12; -x_46 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; -lean_inc(x_38); -x_47 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_47, 0, x_38); -lean_ctor_set(x_47, 1, x_45); -lean_ctor_set(x_47, 2, x_46); -x_48 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; -lean_inc(x_38); -lean_ctor_set_tag(x_41, 2); -lean_ctor_set(x_41, 1, x_48); -lean_ctor_set(x_41, 0, x_38); -x_49 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; -lean_inc(x_38); -x_50 = l_Lean_Syntax_node1(x_38, x_49, x_41); -lean_inc(x_38); -x_51 = l_Lean_Syntax_node1(x_38, x_45, x_50); -lean_inc_n(x_47, 4); -x_52 = l_Lean_Syntax_node6(x_38, x_2, x_47, x_47, x_47, x_51, x_47, x_47); -x_53 = lean_apply_4(x_3, x_52, x_8, x_9, x_43); -return x_53; +x_35 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__3(x_13, x_1, x_2, x_11, x_33, x_5, x_6, x_7, x_8, x_34); +lean_dec(x_33); +return x_35; } 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; -x_54 = lean_ctor_get(x_41, 1); -lean_inc(x_54); -lean_dec(x_41); -x_55 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__12; -x_56 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; -lean_inc(x_38); -x_57 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_57, 0, x_38); -lean_ctor_set(x_57, 1, x_55); -lean_ctor_set(x_57, 2, x_56); -x_58 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; -lean_inc(x_38); -x_59 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_59, 0, x_38); -lean_ctor_set(x_59, 1, x_58); -x_60 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; -lean_inc(x_38); -x_61 = l_Lean_Syntax_node1(x_38, x_60, x_59); -lean_inc(x_38); -x_62 = l_Lean_Syntax_node1(x_38, x_55, x_61); -lean_inc_n(x_57, 4); -x_63 = l_Lean_Syntax_node6(x_38, x_2, x_57, x_57, x_57, x_62, x_57, x_57); -x_64 = lean_apply_4(x_3, x_63, x_8, x_9, x_54); -return x_64; +lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_36 = lean_ctor_get(x_16, 1); +lean_inc(x_36); +lean_dec(x_16); +lean_inc(x_13); +x_37 = lean_array_to_list(x_13); +x_38 = lean_box(0); +x_39 = l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__12(x_37, x_38); +x_40 = l_Lean_MessageData_ofList(x_39); +x_41 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__4___closed__2; +x_42 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_42, 0, x_41); +lean_ctor_set(x_42, 1, x_40); +x_43 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +x_44 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_44, 0, x_42); +lean_ctor_set(x_44, 1, x_43); +x_45 = l_Lean_addTrace___at_Lean_Meta_processPostponed_loop___spec__2(x_15, x_44, x_5, x_6, x_7, x_8, x_36); +x_46 = lean_ctor_get(x_45, 0); +lean_inc(x_46); +x_47 = lean_ctor_get(x_45, 1); +lean_inc(x_47); +lean_dec(x_45); +x_48 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__3(x_13, x_1, x_2, x_11, x_46, x_5, x_6, x_7, x_8, x_47); +lean_dec(x_46); +return x_48; +} } } else { -lean_object* x_65; lean_object* x_66; uint8_t x_67; -x_65 = lean_unsigned_to_nat(5u); -x_66 = l_Lean_Syntax_getArg(x_1, x_65); -x_67 = l_Lean_Syntax_matchesNull(x_66, x_13); -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; 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; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; uint8_t x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; uint8_t x_95; +uint8_t x_49; +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); -x_68 = l_Lean_Elab_Command_getRef(x_8, x_9, x_10); -x_69 = lean_ctor_get(x_68, 0); -lean_inc(x_69); -x_70 = lean_ctor_get(x_68, 1); -lean_inc(x_70); -lean_dec(x_68); -x_71 = l_Lean_replaceRef(x_1, x_69); -lean_dec(x_69); -x_72 = lean_ctor_get(x_8, 0); -lean_inc(x_72); -x_73 = lean_ctor_get(x_8, 1); -lean_inc(x_73); -x_74 = lean_ctor_get(x_8, 2); -lean_inc(x_74); -x_75 = lean_ctor_get(x_8, 3); -lean_inc(x_75); -x_76 = lean_ctor_get(x_8, 4); -lean_inc(x_76); -x_77 = lean_ctor_get(x_8, 5); -lean_inc(x_77); -x_78 = lean_ctor_get(x_8, 7); -lean_inc(x_78); -x_79 = lean_ctor_get(x_8, 8); -lean_inc(x_79); -x_80 = lean_ctor_get(x_8, 9); -lean_inc(x_80); -x_81 = lean_ctor_get_uint8(x_8, sizeof(void*)*10); -x_82 = lean_alloc_ctor(0, 10, 1); -lean_ctor_set(x_82, 0, x_72); -lean_ctor_set(x_82, 1, x_73); -lean_ctor_set(x_82, 2, x_74); -lean_ctor_set(x_82, 3, x_75); -lean_ctor_set(x_82, 4, x_76); -lean_ctor_set(x_82, 5, x_77); -lean_ctor_set(x_82, 6, x_71); -lean_ctor_set(x_82, 7, x_78); -lean_ctor_set(x_82, 8, x_79); -lean_ctor_set(x_82, 9, x_80); -lean_ctor_set_uint8(x_82, sizeof(void*)*10, x_81); -x_83 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__3; -x_84 = 2; -x_85 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_83, x_84, x_82, x_9, x_70); -x_86 = lean_ctor_get(x_85, 1); -lean_inc(x_86); -lean_dec(x_85); -x_87 = l_Lean_Elab_Command_getRef(x_8, x_9, x_86); -x_88 = lean_ctor_get(x_87, 0); -lean_inc(x_88); -x_89 = lean_ctor_get(x_87, 1); -lean_inc(x_89); -lean_dec(x_87); -x_90 = 0; -x_91 = l_Lean_SourceInfo_fromRef(x_88, x_90); -lean_dec(x_88); -x_92 = l_Lean_Elab_Command_getCurrMacroScope(x_8, x_9, x_89); -x_93 = lean_ctor_get(x_92, 1); -lean_inc(x_93); -lean_dec(x_92); -x_94 = l_Lean_Elab_Command_getMainModule___rarg(x_9, x_93); -x_95 = !lean_is_exclusive(x_94); -if (x_95 == 0) +lean_dec(x_2); +lean_dec(x_1); +x_49 = !lean_is_exclusive(x_12); +if (x_49 == 0) { -lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; -x_96 = lean_ctor_get(x_94, 1); -x_97 = lean_ctor_get(x_94, 0); -lean_dec(x_97); -x_98 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__12; -x_99 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; -lean_inc(x_91); -x_100 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_100, 0, x_91); -lean_ctor_set(x_100, 1, x_98); -lean_ctor_set(x_100, 2, x_99); -x_101 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; -lean_inc(x_91); -lean_ctor_set_tag(x_94, 2); -lean_ctor_set(x_94, 1, x_101); -lean_ctor_set(x_94, 0, x_91); -x_102 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; -lean_inc(x_91); -x_103 = l_Lean_Syntax_node1(x_91, x_102, x_94); -lean_inc(x_91); -x_104 = l_Lean_Syntax_node1(x_91, x_98, x_103); -lean_inc_n(x_100, 4); -x_105 = l_Lean_Syntax_node6(x_91, x_2, x_100, x_100, x_100, x_104, x_100, x_100); -x_106 = lean_apply_4(x_3, x_105, x_8, x_9, x_96); -return x_106; +return x_12; } else { -lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; -x_107 = lean_ctor_get(x_94, 1); -lean_inc(x_107); -lean_dec(x_94); -x_108 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__12; -x_109 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; -lean_inc(x_91); -x_110 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_110, 0, x_91); -lean_ctor_set(x_110, 1, x_108); -lean_ctor_set(x_110, 2, x_109); -x_111 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; -lean_inc(x_91); -x_112 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_112, 0, x_91); -lean_ctor_set(x_112, 1, x_111); -x_113 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; -lean_inc(x_91); -x_114 = l_Lean_Syntax_node1(x_91, x_113, x_112); -lean_inc(x_91); -x_115 = l_Lean_Syntax_node1(x_91, x_108, x_114); -lean_inc_n(x_110, 4); -x_116 = l_Lean_Syntax_node6(x_91, x_2, x_110, x_110, x_110, x_115, x_110, x_110); -x_117 = lean_apply_4(x_3, x_116, x_8, x_9, x_107); -return x_117; +lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_50 = lean_ctor_get(x_12, 0); +x_51 = lean_ctor_get(x_12, 1); +lean_inc(x_51); +lean_inc(x_50); +lean_dec(x_12); +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 +} +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___closed__1() { +_start: { -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; uint8_t x_126; -x_118 = l_Lean_Elab_Command_getRef(x_8, x_9, x_10); -x_119 = lean_ctor_get(x_118, 0); -lean_inc(x_119); -x_120 = lean_ctor_get(x_118, 1); -lean_inc(x_120); -lean_dec(x_118); -x_121 = 0; -x_122 = l_Lean_SourceInfo_fromRef(x_119, x_121); -lean_dec(x_119); -x_123 = l_Lean_Elab_Command_getCurrMacroScope(x_8, x_9, x_120); -x_124 = lean_ctor_get(x_123, 1); -lean_inc(x_124); -lean_dec(x_123); -x_125 = l_Lean_Elab_Command_getMainModule___rarg(x_9, x_124); -x_126 = !lean_is_exclusive(x_125); -if (x_126 == 0) +lean_object* x_1; +x_1 = l_Lean_Elab_Command_inductive_autoPromoteIndices; +return x_1; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams(lean_object* x_1, lean_object* x_2, lean_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_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_127 = lean_ctor_get(x_125, 1); -x_128 = lean_ctor_get(x_125, 0); -lean_dec(x_128); -x_129 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; -lean_inc(x_122); -lean_ctor_set_tag(x_125, 2); -lean_ctor_set(x_125, 1, x_129); -lean_ctor_set(x_125, 0, x_122); -x_130 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; -lean_inc(x_122); -x_131 = l_Lean_Syntax_node1(x_122, x_130, x_125); -x_132 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__12; -lean_inc(x_122); -x_133 = l_Lean_Syntax_node1(x_122, x_132, x_131); -x_134 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; -lean_inc(x_122); -x_135 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_135, 0, x_122); -lean_ctor_set(x_135, 1, x_132); -lean_ctor_set(x_135, 2, x_134); -if (lean_obj_tag(x_6) == 0) +lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_9 = lean_ctor_get(x_6, 2); +lean_inc(x_9); +x_10 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___closed__1; +x_11 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_9, x_10); +lean_dec(x_9); +if (x_11 == 0) { -x_136 = x_134; -goto block_163; +lean_object* x_12; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_12 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_1); +lean_ctor_set(x_12, 1, x_8); +return x_12; } else { -lean_object* x_164; lean_object* x_165; -x_164 = lean_ctor_get(x_6, 0); -lean_inc(x_164); -lean_dec(x_6); -x_165 = l_Array_mkArray1___rarg(x_164); -x_136 = x_165; -goto block_163; +lean_object* x_13; lean_object* x_14; +x_13 = lean_box(0); +x_14 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__4(x_2, x_1, x_3, x_13, x_4, x_5, x_6, x_7, x_8); +return x_14; } -block_163: -{ -lean_object* x_137; lean_object* x_138; -x_137 = l_Array_append___rarg(x_134, x_136); -lean_dec(x_136); -lean_inc(x_122); -x_138 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_138, 0, x_122); -lean_ctor_set(x_138, 1, x_132); -lean_ctor_set(x_138, 2, x_137); -if (lean_obj_tag(x_4) == 0) +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___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_139; lean_object* x_140; -x_139 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__6; -lean_inc(x_122); -x_140 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_140, 0, x_122); -lean_ctor_set(x_140, 1, x_132); -lean_ctor_set(x_140, 2, x_139); -if (lean_obj_tag(x_5) == 0) +size_t x_11; size_t x_12; lean_object* x_13; +x_11 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_12 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_13 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__1(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: { -lean_object* x_141; lean_object* x_142; -lean_inc(x_135); -lean_inc(x_140); -x_141 = l_Lean_Syntax_node6(x_122, x_2, x_138, x_140, x_140, x_133, x_135, x_135); -x_142 = lean_apply_4(x_3, x_141, x_8, x_9, x_127); -return x_142; +size_t x_10; size_t x_11; lean_object* x_12; +x_10 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_11 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_12 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__2(x_1, x_10, x_11, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_1); +return x_12; } -else +} +LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___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_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; -x_143 = lean_ctor_get(x_5, 0); -lean_inc(x_143); -lean_dec(x_5); -x_144 = l_Array_mkArray1___rarg(x_143); -x_145 = l_Array_append___rarg(x_134, x_144); -lean_dec(x_144); -lean_inc(x_122); -x_146 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_146, 0, x_122); -lean_ctor_set(x_146, 1, x_132); -lean_ctor_set(x_146, 2, x_145); -lean_inc(x_135); -x_147 = l_Lean_Syntax_node6(x_122, x_2, x_138, x_140, x_146, x_133, x_135, x_135); -x_148 = lean_apply_4(x_3, x_147, x_8, x_9, x_127); -return x_148; +lean_object* x_9; +x_9 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_1); +return x_9; } } -else +LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: { -lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; -x_149 = lean_ctor_get(x_4, 0); -lean_inc(x_149); -lean_dec(x_4); -x_150 = l_Array_mkArray1___rarg(x_149); -x_151 = l_Array_append___rarg(x_134, x_150); -lean_dec(x_150); -lean_inc(x_122); -x_152 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_152, 0, x_122); -lean_ctor_set(x_152, 1, x_132); -lean_ctor_set(x_152, 2, x_151); -if (lean_obj_tag(x_5) == 0) -{ -lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; -x_153 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__6; -lean_inc(x_122); -x_154 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_154, 0, x_122); -lean_ctor_set(x_154, 1, x_132); -lean_ctor_set(x_154, 2, x_153); -lean_inc(x_135); -x_155 = l_Lean_Syntax_node6(x_122, x_2, x_138, x_152, x_154, x_133, x_135, x_135); -x_156 = lean_apply_4(x_3, x_155, x_8, x_9, x_127); -return x_156; +lean_object* x_9; +x_9 = l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_1); +return x_9; } -else +} +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: { -lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; -x_157 = lean_ctor_get(x_5, 0); -lean_inc(x_157); -lean_dec(x_5); -x_158 = l_Array_mkArray1___rarg(x_157); -x_159 = l_Array_append___rarg(x_134, x_158); -lean_dec(x_158); -lean_inc(x_122); -x_160 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_160, 0, x_122); -lean_ctor_set(x_160, 1, x_132); -lean_ctor_set(x_160, 2, x_159); -lean_inc(x_135); -x_161 = l_Lean_Syntax_node6(x_122, x_2, x_138, x_152, x_160, x_133, x_135, x_135); -x_162 = lean_apply_4(x_3, x_161, x_8, x_9, x_127); -return x_162; +uint8_t x_5; size_t x_6; size_t x_7; uint8_t x_8; lean_object* x_9; +x_5 = lean_unbox(x_1); +lean_dec(x_1); +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_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__7(x_5, x_2, x_6, x_7); +lean_dec(x_2); +x_9 = lean_box(x_8); +return x_9; } } +LEAN_EXPORT lean_object* l_Array_contains___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__6___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +uint8_t x_3; uint8_t x_4; lean_object* x_5; +x_3 = lean_unbox(x_2); +lean_dec(x_2); +x_4 = l_Array_contains___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__6(x_1, x_3); +lean_dec(x_1); +x_5 = lean_box(x_4); +return x_5; } } -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; -x_166 = lean_ctor_get(x_125, 1); -lean_inc(x_166); -lean_dec(x_125); -x_167 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; -lean_inc(x_122); -x_168 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_168, 0, x_122); -lean_ctor_set(x_168, 1, x_167); -x_169 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; -lean_inc(x_122); -x_170 = l_Lean_Syntax_node1(x_122, x_169, x_168); -x_171 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__12; -lean_inc(x_122); -x_172 = l_Lean_Syntax_node1(x_122, x_171, x_170); -x_173 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; -lean_inc(x_122); -x_174 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_174, 0, x_122); -lean_ctor_set(x_174, 1, x_171); -lean_ctor_set(x_174, 2, x_173); -if (lean_obj_tag(x_6) == 0) +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: { -x_175 = x_173; -goto block_202; +size_t x_4; size_t x_5; uint8_t x_6; lean_object* x_7; +x_4 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_5 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_6 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__8(x_1, x_4, x_5); +lean_dec(x_1); +x_7 = lean_box(x_6); +return x_7; } -else +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, 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_203; lean_object* x_204; -x_203 = lean_ctor_get(x_6, 0); -lean_inc(x_203); +size_t x_13; lean_object* x_14; +x_13 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_14 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__1(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_6); -x_204 = l_Array_mkArray1___rarg(x_203); -x_175 = x_204; -goto block_202; +return x_14; } -block_202: -{ -lean_object* x_176; lean_object* x_177; -x_176 = l_Array_append___rarg(x_173, x_175); -lean_dec(x_175); -lean_inc(x_122); -x_177 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_177, 0, x_122); -lean_ctor_set(x_177, 1, x_171); -lean_ctor_set(x_177, 2, x_176); -if (lean_obj_tag(x_4) == 0) -{ -lean_object* x_178; lean_object* x_179; -x_178 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__6; -lean_inc(x_122); -x_179 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_179, 0, x_122); -lean_ctor_set(x_179, 1, x_171); -lean_ctor_set(x_179, 2, x_178); -if (lean_obj_tag(x_5) == 0) -{ -lean_object* x_180; lean_object* x_181; -lean_inc(x_174); -lean_inc(x_179); -x_180 = l_Lean_Syntax_node6(x_122, x_2, x_177, x_179, x_179, x_172, x_174, x_174); -x_181 = lean_apply_4(x_3, x_180, x_8, x_9, x_166); -return x_181; } -else +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___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_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; -x_182 = lean_ctor_get(x_5, 0); -lean_inc(x_182); +size_t x_11; lean_object* x_12; +x_11 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_12 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__2(x_1, x_2, x_3, x_11, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_5); -x_183 = l_Array_mkArray1___rarg(x_182); -x_184 = l_Array_append___rarg(x_173, x_183); -lean_dec(x_183); -lean_inc(x_122); -x_185 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_185, 0, x_122); -lean_ctor_set(x_185, 1, x_171); -lean_ctor_set(x_185, 2, x_184); -lean_inc(x_174); -x_186 = l_Lean_Syntax_node6(x_122, x_2, x_177, x_179, x_185, x_172, x_174, x_174); -x_187 = lean_apply_4(x_3, x_186, x_8, x_9, x_166); -return x_187; +return x_12; } } -else +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: { -lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; -x_188 = lean_ctor_get(x_4, 0); -lean_inc(x_188); +size_t x_11; lean_object* x_12; +x_11 = lean_unbox_usize(x_4); lean_dec(x_4); -x_189 = l_Array_mkArray1___rarg(x_188); -x_190 = l_Array_append___rarg(x_173, x_189); -lean_dec(x_189); -lean_inc(x_122); -x_191 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_191, 0, x_122); -lean_ctor_set(x_191, 1, x_171); -lean_ctor_set(x_191, 2, x_190); -if (lean_obj_tag(x_5) == 0) -{ -lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; -x_192 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__6; -lean_inc(x_122); -x_193 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_193, 0, x_122); -lean_ctor_set(x_193, 1, x_171); -lean_ctor_set(x_193, 2, x_192); -lean_inc(x_174); -x_194 = l_Lean_Syntax_node6(x_122, x_2, x_177, x_191, x_193, x_172, x_174, x_174); -x_195 = lean_apply_4(x_3, x_194, x_8, x_9, x_166); -return x_195; -} -else -{ -lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; -x_196 = lean_ctor_get(x_5, 0); -lean_inc(x_196); +x_12 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__3(x_1, x_2, x_3, x_11, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_5); -x_197 = l_Array_mkArray1___rarg(x_196); -x_198 = l_Array_append___rarg(x_173, x_197); -lean_dec(x_197); -lean_inc(x_122); -x_199 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_199, 0, x_122); -lean_ctor_set(x_199, 1, x_171); -lean_ctor_set(x_199, 2, x_198); -lean_inc(x_174); -x_200 = l_Lean_Syntax_node6(x_122, x_2, x_177, x_191, x_199, x_172, x_174, x_174); -x_201 = lean_apply_4(x_3, x_200, x_8, x_9, x_166); -return x_201; +return x_12; } } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__4(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_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18) { +_start: +{ +uint8_t x_19; +x_19 = lean_nat_dec_le(x_9, x_8); +if (x_19 == 0) +{ +lean_object* x_20; uint8_t x_21; +x_20 = lean_unsigned_to_nat(0u); +x_21 = lean_nat_dec_eq(x_7, x_20); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_30; uint8_t x_31; uint8_t x_32; lean_object* x_33; +x_22 = lean_unsigned_to_nat(1u); +x_23 = lean_nat_sub(x_7, x_22); +lean_dec(x_7); +x_30 = lean_array_get_size(x_5); +x_31 = lean_nat_dec_lt(x_8, x_30); +lean_dec(x_30); +x_32 = lean_nat_dec_lt(x_8, x_6); +if (x_31 == 0) +{ +lean_object* x_109; lean_object* x_110; +x_109 = l_Lean_instInhabitedExpr; +x_110 = l_outOfBounds___rarg(x_109); +x_33 = x_110; +goto block_108; } +else +{ +lean_object* x_111; +x_111 = lean_array_fget(x_5, x_8); +x_33 = x_111; +goto block_108; } +block_29: +{ +lean_object* x_26; lean_object* x_27; +x_26 = lean_ctor_get(x_24, 0); +lean_inc(x_26); +lean_dec(x_24); +x_27 = lean_nat_add(x_8, x_10); +lean_dec(x_8); +x_7 = x_23; +x_8 = x_27; +x_11 = x_26; +x_18 = x_25; +goto _start; } +block_108: +{ +lean_object* x_34; +if (x_32 == 0) +{ +lean_object* x_105; lean_object* x_106; +x_105 = l_Lean_Elab_Command_instInhabitedInductiveView; +x_106 = l_outOfBounds___rarg(x_105); +x_34 = x_106; +goto block_104; } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: +else { -lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_11 = lean_unsigned_to_nat(3u); -x_12 = l_Lean_Syntax_getArg(x_1, x_11); -x_13 = l_Lean_Syntax_isNone(x_12); -if (x_13 == 0) +lean_object* x_107; +x_107 = lean_array_fget(x_1, x_8); +x_34 = x_107; +goto block_104; +} +block_104: { -lean_object* x_14; uint8_t x_15; -x_14 = lean_unsigned_to_nat(1u); +lean_object* x_35; lean_object* x_36; +x_35 = lean_ctor_get(x_34, 1); +lean_inc(x_35); +lean_dec(x_34); +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_15 = l_Lean_Syntax_matchesNull(x_12, x_14); -if (x_15 == 0) +lean_inc(x_33); +x_36 = l_Lean_Elab_Term_addLocalVarInfo(x_35, x_33, x_12, x_13, x_14, x_15, x_16, x_17, x_18); +if (lean_obj_tag(x_36) == 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; uint8_t x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; uint8_t x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; -lean_dec(x_12); -lean_dec(x_7); -lean_dec(x_5); -lean_dec(x_4); -x_16 = l_Lean_Elab_Command_getRef(x_8, x_9, x_10); -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_16, 1); -lean_inc(x_18); -lean_dec(x_16); -x_19 = l_Lean_replaceRef(x_1, x_17); -lean_dec(x_17); -x_20 = lean_ctor_get(x_8, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_8, 1); -lean_inc(x_21); -x_22 = lean_ctor_get(x_8, 2); -lean_inc(x_22); -x_23 = lean_ctor_get(x_8, 3); -lean_inc(x_23); -x_24 = lean_ctor_get(x_8, 4); -lean_inc(x_24); -x_25 = lean_ctor_get(x_8, 5); -lean_inc(x_25); -x_26 = lean_ctor_get(x_8, 7); -lean_inc(x_26); -x_27 = lean_ctor_get(x_8, 8); -lean_inc(x_27); -x_28 = lean_ctor_get(x_8, 9); -lean_inc(x_28); -x_29 = lean_ctor_get_uint8(x_8, sizeof(void*)*10); -x_30 = lean_alloc_ctor(0, 10, 1); -lean_ctor_set(x_30, 0, x_20); -lean_ctor_set(x_30, 1, x_21); -lean_ctor_set(x_30, 2, x_22); -lean_ctor_set(x_30, 3, x_23); -lean_ctor_set(x_30, 4, x_24); -lean_ctor_set(x_30, 5, x_25); -lean_ctor_set(x_30, 6, x_19); -lean_ctor_set(x_30, 7, x_26); -lean_ctor_set(x_30, 8, x_27); -lean_ctor_set(x_30, 9, x_28); -lean_ctor_set_uint8(x_30, sizeof(void*)*10, x_29); -x_31 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__3; -x_32 = 2; -x_33 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_31, x_32, x_30, x_9, x_18); -x_34 = lean_ctor_get(x_33, 1); -lean_inc(x_34); -lean_dec(x_33); -x_35 = l_Lean_Elab_Command_getRef(x_8, x_9, x_34); -x_36 = lean_ctor_get(x_35, 0); -lean_inc(x_36); -x_37 = lean_ctor_get(x_35, 1); +lean_object* x_37; uint8_t x_38; +x_37 = lean_ctor_get(x_36, 1); lean_inc(x_37); -lean_dec(x_35); -x_38 = 0; -x_39 = l_Lean_SourceInfo_fromRef(x_36, x_38); lean_dec(x_36); -x_40 = l_Lean_Elab_Command_getCurrMacroScope(x_8, x_9, x_37); -x_41 = lean_ctor_get(x_40, 1); -lean_inc(x_41); -lean_dec(x_40); -x_42 = l_Lean_Elab_Command_getMainModule___rarg(x_9, x_41); -x_43 = !lean_is_exclusive(x_42); -if (x_43 == 0) +x_38 = lean_nat_dec_lt(x_8, x_3); +if (x_38 == 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_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; uint8_t x_48; uint8_t x_49; lean_object* x_50; +x_39 = l_Lean_Elab_Command_instInhabitedElabHeaderResult; +x_40 = l_outOfBounds___rarg(x_39); +x_41 = lean_ctor_get(x_40, 5); +lean_inc(x_41); +x_42 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_41, x_12, x_13, x_14, x_15, x_16, x_17, x_37); +x_43 = lean_ctor_get(x_42, 0); +lean_inc(x_43); x_44 = lean_ctor_get(x_42, 1); -x_45 = lean_ctor_get(x_42, 0); +lean_inc(x_44); +lean_dec(x_42); +x_45 = lean_ctor_get(x_40, 4); +lean_inc(x_45); +x_46 = l_Lean_Expr_replaceFVars(x_43, x_45, x_4); lean_dec(x_45); -x_46 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__12; -x_47 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; -lean_inc(x_39); -x_48 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_48, 0, x_39); -lean_ctor_set(x_48, 1, x_46); -lean_ctor_set(x_48, 2, x_47); -x_49 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; -lean_inc(x_39); -lean_ctor_set_tag(x_42, 2); -lean_ctor_set(x_42, 1, x_49); -lean_ctor_set(x_42, 0, x_39); -x_50 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; -lean_inc(x_39); -x_51 = l_Lean_Syntax_node1(x_39, x_50, x_42); -lean_inc(x_39); -x_52 = l_Lean_Syntax_node1(x_39, x_46, x_51); -lean_inc_n(x_48, 4); -x_53 = l_Lean_Syntax_node6(x_39, x_2, x_48, x_48, x_48, x_52, x_48, x_48); -x_54 = lean_apply_4(x_3, x_53, x_8, x_9, x_44); +lean_dec(x_43); +x_47 = 0; +x_48 = 1; +x_49 = 1; +lean_inc(x_4); +x_50 = l_Lean_Meta_mkForallFVars(x_4, x_46, x_47, x_48, x_49, x_14, x_15, x_16, x_17, x_44); +if (lean_obj_tag(x_50) == 0) +{ +lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_51 = lean_ctor_get(x_50, 0); +lean_inc(x_51); +x_52 = lean_ctor_get(x_50, 1); +lean_inc(x_52); +lean_dec(x_50); +lean_inc(x_40); +lean_inc(x_4); +lean_inc(x_5); +x_53 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors), 11, 4); +lean_closure_set(x_53, 0, x_5); +lean_closure_set(x_53, 1, x_33); +lean_closure_set(x_53, 2, x_4); +lean_closure_set(x_53, 3, x_40); +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_54 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___rarg(x_4, x_53, x_12, x_13, x_14, x_15, x_16, x_17, x_52); +if (lean_obj_tag(x_54) == 0) +{ +lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; +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_40, 0); +lean_inc(x_57); +lean_dec(x_40); +x_58 = lean_ctor_get(x_57, 4); +lean_inc(x_58); +lean_dec(x_57); +x_59 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_59, 0, x_58); +lean_ctor_set(x_59, 1, x_51); +lean_ctor_set(x_59, 2, x_55); +x_60 = lean_array_push(x_11, x_59); +x_61 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_61, 0, x_60); +x_24 = x_61; +x_25 = x_56; +goto block_29; +} +else +{ +uint8_t x_62; +lean_dec(x_51); +lean_dec(x_40); +lean_dec(x_23); +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_8); +lean_dec(x_5); +lean_dec(x_4); +x_62 = !lean_is_exclusive(x_54); +if (x_62 == 0) +{ return x_54; } else { -lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; -x_55 = lean_ctor_get(x_42, 1); -lean_inc(x_55); -lean_dec(x_42); -x_56 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__12; -x_57 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; -lean_inc(x_39); -x_58 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_58, 0, x_39); -lean_ctor_set(x_58, 1, x_56); -lean_ctor_set(x_58, 2, x_57); -x_59 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; -lean_inc(x_39); -x_60 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_60, 0, x_39); -lean_ctor_set(x_60, 1, x_59); -x_61 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; -lean_inc(x_39); -x_62 = l_Lean_Syntax_node1(x_39, x_61, x_60); -lean_inc(x_39); -x_63 = l_Lean_Syntax_node1(x_39, x_56, x_62); -lean_inc_n(x_58, 4); -x_64 = l_Lean_Syntax_node6(x_39, x_2, x_58, x_58, x_58, x_63, x_58, x_58); -x_65 = lean_apply_4(x_3, x_64, x_8, x_9, x_55); +lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_63 = lean_ctor_get(x_54, 0); +x_64 = lean_ctor_get(x_54, 1); +lean_inc(x_64); +lean_inc(x_63); +lean_dec(x_54); +x_65 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_65, 0, x_63); +lean_ctor_set(x_65, 1, x_64); return x_65; } } +} else { -lean_object* x_66; lean_object* x_67; lean_object* x_68; uint8_t x_69; -x_66 = lean_unsigned_to_nat(0u); -x_67 = l_Lean_Syntax_getArg(x_12, x_66); +uint8_t x_66; +lean_dec(x_40); +lean_dec(x_33); +lean_dec(x_23); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); lean_dec(x_12); -x_68 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; -x_69 = l_Lean_Syntax_isOfKind(x_67, 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; uint8_t x_83; lean_object* x_84; lean_object* x_85; uint8_t x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; uint8_t x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; uint8_t x_97; -lean_dec(x_7); +lean_dec(x_11); +lean_dec(x_8); lean_dec(x_5); lean_dec(x_4); -x_70 = l_Lean_Elab_Command_getRef(x_8, x_9, x_10); -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_replaceRef(x_1, x_71); -lean_dec(x_71); -x_74 = lean_ctor_get(x_8, 0); -lean_inc(x_74); -x_75 = lean_ctor_get(x_8, 1); +x_66 = !lean_is_exclusive(x_50); +if (x_66 == 0) +{ +return x_50; +} +else +{ +lean_object* x_67; lean_object* x_68; lean_object* x_69; +x_67 = lean_ctor_get(x_50, 0); +x_68 = lean_ctor_get(x_50, 1); +lean_inc(x_68); +lean_inc(x_67); +lean_dec(x_50); +x_69 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_69, 0, x_67); +lean_ctor_set(x_69, 1, x_68); +return x_69; +} +} +} +else +{ +lean_object* x_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; uint8_t x_78; uint8_t x_79; lean_object* x_80; +x_70 = lean_array_fget(x_2, x_8); +x_71 = lean_ctor_get(x_70, 5); +lean_inc(x_71); +x_72 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_71, x_12, x_13, x_14, x_15, x_16, x_17, x_37); +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_70, 4); lean_inc(x_75); -x_76 = lean_ctor_get(x_8, 2); -lean_inc(x_76); -x_77 = lean_ctor_get(x_8, 3); -lean_inc(x_77); -x_78 = lean_ctor_get(x_8, 4); -lean_inc(x_78); -x_79 = lean_ctor_get(x_8, 5); -lean_inc(x_79); -x_80 = lean_ctor_get(x_8, 7); -lean_inc(x_80); -x_81 = lean_ctor_get(x_8, 8); +x_76 = l_Lean_Expr_replaceFVars(x_73, x_75, x_4); +lean_dec(x_75); +lean_dec(x_73); +x_77 = 0; +x_78 = 1; +x_79 = 1; +lean_inc(x_4); +x_80 = l_Lean_Meta_mkForallFVars(x_4, x_76, x_77, x_78, x_79, x_14, x_15, x_16, x_17, x_74); +if (lean_obj_tag(x_80) == 0) +{ +lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; +x_81 = lean_ctor_get(x_80, 0); lean_inc(x_81); -x_82 = lean_ctor_get(x_8, 9); +x_82 = lean_ctor_get(x_80, 1); lean_inc(x_82); -x_83 = lean_ctor_get_uint8(x_8, sizeof(void*)*10); -x_84 = lean_alloc_ctor(0, 10, 1); -lean_ctor_set(x_84, 0, x_74); -lean_ctor_set(x_84, 1, x_75); -lean_ctor_set(x_84, 2, x_76); -lean_ctor_set(x_84, 3, x_77); -lean_ctor_set(x_84, 4, x_78); -lean_ctor_set(x_84, 5, x_79); -lean_ctor_set(x_84, 6, x_73); -lean_ctor_set(x_84, 7, x_80); -lean_ctor_set(x_84, 8, x_81); -lean_ctor_set(x_84, 9, x_82); -lean_ctor_set_uint8(x_84, sizeof(void*)*10, x_83); -x_85 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__3; -x_86 = 2; -x_87 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_85, x_86, x_84, x_9, x_72); -x_88 = lean_ctor_get(x_87, 1); +lean_dec(x_80); +lean_inc(x_70); +lean_inc(x_4); +lean_inc(x_5); +x_83 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors), 11, 4); +lean_closure_set(x_83, 0, x_5); +lean_closure_set(x_83, 1, x_33); +lean_closure_set(x_83, 2, x_4); +lean_closure_set(x_83, 3, x_70); +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_84 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withExplicitToImplicit___rarg(x_4, x_83, x_12, x_13, x_14, x_15, x_16, x_17, x_82); +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; lean_object* x_90; lean_object* x_91; +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_70, 0); +lean_inc(x_87); +lean_dec(x_70); +x_88 = lean_ctor_get(x_87, 4); lean_inc(x_88); lean_dec(x_87); -x_89 = l_Lean_Elab_Command_getRef(x_8, x_9, 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); -x_92 = 0; -x_93 = l_Lean_SourceInfo_fromRef(x_90, x_92); -lean_dec(x_90); -x_94 = l_Lean_Elab_Command_getCurrMacroScope(x_8, x_9, x_91); -x_95 = lean_ctor_get(x_94, 1); -lean_inc(x_95); -lean_dec(x_94); -x_96 = l_Lean_Elab_Command_getMainModule___rarg(x_9, x_95); -x_97 = !lean_is_exclusive(x_96); -if (x_97 == 0) -{ -lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; -x_98 = lean_ctor_get(x_96, 1); -x_99 = lean_ctor_get(x_96, 0); -lean_dec(x_99); -x_100 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__12; -x_101 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; -lean_inc(x_93); -x_102 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_102, 0, x_93); -lean_ctor_set(x_102, 1, x_100); -lean_ctor_set(x_102, 2, x_101); -x_103 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; -lean_inc(x_93); -lean_ctor_set_tag(x_96, 2); -lean_ctor_set(x_96, 1, x_103); -lean_ctor_set(x_96, 0, x_93); -lean_inc(x_93); -x_104 = l_Lean_Syntax_node1(x_93, x_68, x_96); -lean_inc(x_93); -x_105 = l_Lean_Syntax_node1(x_93, x_100, x_104); -lean_inc_n(x_102, 4); -x_106 = l_Lean_Syntax_node6(x_93, x_2, x_102, x_102, x_102, x_105, x_102, x_102); -x_107 = lean_apply_4(x_3, x_106, x_8, x_9, x_98); -return x_107; +x_89 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_89, 0, x_88); +lean_ctor_set(x_89, 1, x_81); +lean_ctor_set(x_89, 2, x_85); +x_90 = lean_array_push(x_11, x_89); +x_91 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_91, 0, x_90); +x_24 = x_91; +x_25 = x_86; +goto block_29; } else { -lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; -x_108 = lean_ctor_get(x_96, 1); -lean_inc(x_108); -lean_dec(x_96); -x_109 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__12; -x_110 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; -lean_inc(x_93); -x_111 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_111, 0, x_93); -lean_ctor_set(x_111, 1, x_109); -lean_ctor_set(x_111, 2, x_110); -x_112 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; -lean_inc(x_93); -x_113 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_113, 0, x_93); -lean_ctor_set(x_113, 1, x_112); -lean_inc(x_93); -x_114 = l_Lean_Syntax_node1(x_93, x_68, x_113); -lean_inc(x_93); -x_115 = l_Lean_Syntax_node1(x_93, x_109, x_114); -lean_inc_n(x_111, 4); -x_116 = l_Lean_Syntax_node6(x_93, x_2, x_111, x_111, x_111, x_115, x_111, x_111); -x_117 = lean_apply_4(x_3, x_116, x_8, x_9, x_108); -return x_117; -} +uint8_t x_92; +lean_dec(x_81); +lean_dec(x_70); +lean_dec(x_23); +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_8); +lean_dec(x_5); +lean_dec(x_4); +x_92 = !lean_is_exclusive(x_84); +if (x_92 == 0) +{ +return x_84; } else { -lean_object* x_118; lean_object* x_119; -x_118 = lean_box(0); -x_119 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2(x_1, x_2, x_3, x_4, x_7, x_5, x_118, x_8, x_9, x_10); -return x_119; +lean_object* x_93; lean_object* x_94; lean_object* x_95; +x_93 = lean_ctor_get(x_84, 0); +x_94 = lean_ctor_get(x_84, 1); +lean_inc(x_94); +lean_inc(x_93); +lean_dec(x_84); +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_120; lean_object* x_121; +uint8_t x_96; +lean_dec(x_70); +lean_dec(x_33); +lean_dec(x_23); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); lean_dec(x_12); -x_120 = lean_box(0); -x_121 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2(x_1, x_2, x_3, x_4, x_7, x_5, x_120, x_8, x_9, x_10); -return x_121; -} -} -} -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_10 = lean_unsigned_to_nat(2u); -x_11 = l_Lean_Syntax_getArg(x_1, x_10); -x_12 = l_Lean_Syntax_isNone(x_11); -if (x_12 == 0) -{ -lean_object* x_13; uint8_t x_14; -x_13 = lean_unsigned_to_nat(1u); -lean_inc(x_11); -x_14 = l_Lean_Syntax_matchesNull(x_11, x_13); -if (x_14 == 0) -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t 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; uint8_t x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; lean_dec(x_11); -lean_dec(x_6); +lean_dec(x_8); +lean_dec(x_5); lean_dec(x_4); -x_15 = l_Lean_Elab_Command_getRef(x_7, x_8, x_9); -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_replaceRef(x_1, x_16); -lean_dec(x_16); -x_19 = lean_ctor_get(x_7, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_7, 1); -lean_inc(x_20); -x_21 = lean_ctor_get(x_7, 2); -lean_inc(x_21); -x_22 = lean_ctor_get(x_7, 3); -lean_inc(x_22); -x_23 = lean_ctor_get(x_7, 4); -lean_inc(x_23); -x_24 = lean_ctor_get(x_7, 5); -lean_inc(x_24); -x_25 = lean_ctor_get(x_7, 7); -lean_inc(x_25); -x_26 = lean_ctor_get(x_7, 8); -lean_inc(x_26); -x_27 = lean_ctor_get(x_7, 9); -lean_inc(x_27); -x_28 = lean_ctor_get_uint8(x_7, sizeof(void*)*10); -x_29 = lean_alloc_ctor(0, 10, 1); -lean_ctor_set(x_29, 0, x_19); -lean_ctor_set(x_29, 1, x_20); -lean_ctor_set(x_29, 2, x_21); -lean_ctor_set(x_29, 3, x_22); -lean_ctor_set(x_29, 4, x_23); -lean_ctor_set(x_29, 5, x_24); -lean_ctor_set(x_29, 6, x_18); -lean_ctor_set(x_29, 7, x_25); -lean_ctor_set(x_29, 8, x_26); -lean_ctor_set(x_29, 9, x_27); -lean_ctor_set_uint8(x_29, sizeof(void*)*10, 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; -x_32 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_30, x_31, x_29, x_8, x_17); -x_33 = lean_ctor_get(x_32, 1); -lean_inc(x_33); -lean_dec(x_32); -x_34 = l_Lean_Elab_Command_getRef(x_7, x_8, x_33); -x_35 = lean_ctor_get(x_34, 0); -lean_inc(x_35); -x_36 = lean_ctor_get(x_34, 1); -lean_inc(x_36); -lean_dec(x_34); -x_37 = 0; -x_38 = l_Lean_SourceInfo_fromRef(x_35, x_37); -lean_dec(x_35); -x_39 = l_Lean_Elab_Command_getCurrMacroScope(x_7, x_8, x_36); -x_40 = lean_ctor_get(x_39, 1); -lean_inc(x_40); -lean_dec(x_39); -x_41 = l_Lean_Elab_Command_getMainModule___rarg(x_8, x_40); -x_42 = !lean_is_exclusive(x_41); -if (x_42 == 0) +x_96 = !lean_is_exclusive(x_80); +if (x_96 == 0) { -lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; -x_43 = lean_ctor_get(x_41, 1); -x_44 = lean_ctor_get(x_41, 0); -lean_dec(x_44); -x_45 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__12; -x_46 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; -lean_inc(x_38); -x_47 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_47, 0, x_38); -lean_ctor_set(x_47, 1, x_45); -lean_ctor_set(x_47, 2, x_46); -x_48 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; -lean_inc(x_38); -lean_ctor_set_tag(x_41, 2); -lean_ctor_set(x_41, 1, x_48); -lean_ctor_set(x_41, 0, x_38); -x_49 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; -lean_inc(x_38); -x_50 = l_Lean_Syntax_node1(x_38, x_49, x_41); -lean_inc(x_38); -x_51 = l_Lean_Syntax_node1(x_38, x_45, x_50); -lean_inc_n(x_47, 4); -x_52 = l_Lean_Syntax_node6(x_38, x_2, x_47, x_47, x_47, x_51, x_47, x_47); -x_53 = lean_apply_4(x_3, x_52, x_7, x_8, x_43); -return x_53; +return x_80; } 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; -x_54 = lean_ctor_get(x_41, 1); -lean_inc(x_54); -lean_dec(x_41); -x_55 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__12; -x_56 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; -lean_inc(x_38); -x_57 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_57, 0, x_38); -lean_ctor_set(x_57, 1, x_55); -lean_ctor_set(x_57, 2, x_56); -x_58 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; -lean_inc(x_38); -x_59 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_59, 0, x_38); -lean_ctor_set(x_59, 1, x_58); -x_60 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; -lean_inc(x_38); -x_61 = l_Lean_Syntax_node1(x_38, x_60, x_59); -lean_inc(x_38); -x_62 = l_Lean_Syntax_node1(x_38, x_55, x_61); -lean_inc_n(x_57, 4); -x_63 = l_Lean_Syntax_node6(x_38, x_2, x_57, x_57, x_57, x_62, x_57, x_57); -x_64 = lean_apply_4(x_3, x_63, x_7, x_8, x_54); -return x_64; +lean_object* x_97; lean_object* x_98; lean_object* x_99; +x_97 = lean_ctor_get(x_80, 0); +x_98 = lean_ctor_get(x_80, 1); +lean_inc(x_98); +lean_inc(x_97); +lean_dec(x_80); +x_99 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_99, 0, x_97); +lean_ctor_set(x_99, 1, x_98); +return x_99; +} +} } } else { -lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_65 = lean_unsigned_to_nat(0u); -x_66 = l_Lean_Syntax_getArg(x_11, x_65); +uint8_t x_100; +lean_dec(x_33); +lean_dec(x_23); +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); -x_67 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_67, 0, x_66); -x_68 = lean_box(0); -x_69 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__3(x_1, x_2, x_3, x_6, x_4, x_68, x_67, x_7, x_8, x_9); -return x_69; -} +lean_dec(x_8); +lean_dec(x_5); +lean_dec(x_4); +x_100 = !lean_is_exclusive(x_36); +if (x_100 == 0) +{ +return x_36; } else { -lean_object* x_70; lean_object* x_71; lean_object* x_72; -lean_dec(x_11); -x_70 = lean_box(0); -x_71 = lean_box(0); -x_72 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__3(x_1, x_2, x_3, x_6, x_4, x_71, x_70, x_7, x_8, x_9); -return x_72; +lean_object* x_101; lean_object* x_102; lean_object* x_103; +x_101 = lean_ctor_get(x_36, 0); +x_102 = lean_ctor_get(x_36, 1); +lean_inc(x_102); +lean_inc(x_101); +lean_dec(x_36); +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; } } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__5___closed__1() { -_start: +} +} +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("attributes", 10, 10); -return x_1; +lean_object* x_112; +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_8); +lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_4); +x_112 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_112, 0, x_11); +lean_ctor_set(x_112, 1, x_18); +return x_112; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__5___closed__2() { -_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_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__1; -x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__15; -x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__5___closed__1; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; +lean_object* x_113; +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_8); +lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_4); +x_113 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_113, 0, x_11); +lean_ctor_set(x_113, 1, x_18); +return x_113; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___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_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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_9; lean_object* x_10; uint8_t x_11; -x_9 = lean_unsigned_to_nat(1u); -x_10 = l_Lean_Syntax_getArg(x_1, x_9); -x_11 = l_Lean_Syntax_isNone(x_10); -if (x_11 == 0) -{ -uint8_t x_12; -lean_inc(x_10); -x_12 = l_Lean_Syntax_matchesNull(x_10, x_9); -if (x_12 == 0) +uint8_t x_14; +x_14 = lean_usize_dec_lt(x_5, x_4); +if (x_14 == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t 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_15; +lean_dec(x_12); +lean_dec(x_11); lean_dec(x_10); -lean_dec(x_5); -x_13 = l_Lean_Elab_Command_getRef(x_6, x_7, x_8); -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_replaceRef(x_1, x_14); -lean_dec(x_14); -x_17 = lean_ctor_get(x_6, 0); +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_16; lean_object* x_17; lean_object* x_18; +lean_dec(x_6); +x_16 = lean_array_uget(x_3, x_5); +x_17 = lean_ctor_get(x_16, 2); lean_inc(x_17); -x_18 = lean_ctor_get(x_6, 1); -lean_inc(x_18); -x_19 = lean_ctor_get(x_6, 2); +lean_inc(x_7); +x_18 = l_Lean_mkConstWithLevelParams___at_Lean_Elab_Term_expandDeclId___spec__7(x_17, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +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; uint8_t x_25; lean_object* x_26; +x_19 = lean_ctor_get(x_18, 0); lean_inc(x_19); -x_20 = lean_ctor_get(x_6, 3); +x_20 = lean_ctor_get(x_18, 1); lean_inc(x_20); -x_21 = lean_ctor_get(x_6, 4); +lean_dec(x_18); +x_21 = lean_ctor_get(x_16, 0); lean_inc(x_21); -x_22 = lean_ctor_get(x_6, 5); -lean_inc(x_22); -x_23 = lean_ctor_get(x_6, 7); -lean_inc(x_23); -x_24 = lean_ctor_get(x_6, 8); -lean_inc(x_24); -x_25 = lean_ctor_get(x_6, 9); -lean_inc(x_25); -x_26 = lean_ctor_get_uint8(x_6, sizeof(void*)*10); -x_27 = lean_alloc_ctor(0, 10, 1); -lean_ctor_set(x_27, 0, x_17); -lean_ctor_set(x_27, 1, x_18); -lean_ctor_set(x_27, 2, x_19); -lean_ctor_set(x_27, 3, x_20); -lean_ctor_set(x_27, 4, x_21); -lean_ctor_set(x_27, 5, x_22); -lean_ctor_set(x_27, 6, x_16); -lean_ctor_set(x_27, 7, x_23); -lean_ctor_set(x_27, 8, x_24); -lean_ctor_set(x_27, 9, x_25); -lean_ctor_set_uint8(x_27, sizeof(void*)*10, 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; -x_30 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_28, x_29, x_27, x_7, x_15); -x_31 = lean_ctor_get(x_30, 1); -lean_inc(x_31); -lean_dec(x_30); -x_32 = l_Lean_Elab_Command_getRef(x_6, x_7, 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); -lean_dec(x_32); -x_35 = 0; -x_36 = l_Lean_SourceInfo_fromRef(x_33, x_35); -lean_dec(x_33); -x_37 = l_Lean_Elab_Command_getCurrMacroScope(x_6, x_7, x_34); -x_38 = lean_ctor_get(x_37, 1); -lean_inc(x_38); -lean_dec(x_37); -x_39 = l_Lean_Elab_Command_getMainModule___rarg(x_7, x_38); -x_40 = !lean_is_exclusive(x_39); -if (x_40 == 0) -{ -lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_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_39, 1); -x_42 = lean_ctor_get(x_39, 0); -lean_dec(x_42); -x_43 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__12; -x_44 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; -lean_inc(x_36); -x_45 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_45, 0, x_36); -lean_ctor_set(x_45, 1, x_43); -lean_ctor_set(x_45, 2, x_44); -x_46 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; -lean_inc(x_36); -lean_ctor_set_tag(x_39, 2); -lean_ctor_set(x_39, 1, x_46); -lean_ctor_set(x_39, 0, x_36); -x_47 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; -lean_inc(x_36); -x_48 = l_Lean_Syntax_node1(x_36, x_47, x_39); -lean_inc(x_36); -x_49 = l_Lean_Syntax_node1(x_36, x_43, x_48); -lean_inc_n(x_45, 4); -x_50 = l_Lean_Syntax_node6(x_36, x_2, x_45, x_45, x_45, x_49, x_45, x_45); -x_51 = lean_apply_4(x_3, x_50, x_6, x_7, x_41); -return x_51; -} -else +lean_dec(x_16); +x_22 = lean_unsigned_to_nat(3u); +x_23 = l_Lean_Syntax_getArg(x_21, x_22); +lean_dec(x_21); +x_24 = lean_box(0); +x_25 = 1; +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_2); +lean_inc(x_1); +x_26 = l_Lean_Elab_Term_addTermInfo_x27(x_23, x_19, x_1, x_2, x_24, x_25, x_7, x_8, x_9, x_10, x_11, x_12, x_20); +if (lean_obj_tag(x_26) == 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; -x_52 = lean_ctor_get(x_39, 1); -lean_inc(x_52); -lean_dec(x_39); -x_53 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__12; -x_54 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; -lean_inc(x_36); -x_55 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_55, 0, x_36); -lean_ctor_set(x_55, 1, x_53); -lean_ctor_set(x_55, 2, x_54); -x_56 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; -lean_inc(x_36); -x_57 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_57, 0, x_36); -lean_ctor_set(x_57, 1, x_56); -x_58 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; -lean_inc(x_36); -x_59 = l_Lean_Syntax_node1(x_36, x_58, x_57); -lean_inc(x_36); -x_60 = l_Lean_Syntax_node1(x_36, x_53, x_59); -lean_inc_n(x_55, 4); -x_61 = l_Lean_Syntax_node6(x_36, x_2, x_55, x_55, x_55, x_60, x_55, x_55); -x_62 = lean_apply_4(x_3, x_61, x_6, x_7, x_52); -return x_62; -} +lean_object* x_27; size_t x_28; size_t x_29; lean_object* x_30; +x_27 = lean_ctor_get(x_26, 1); +lean_inc(x_27); +lean_dec(x_26); +x_28 = 1; +x_29 = lean_usize_add(x_5, x_28); +x_30 = lean_box(0); +x_5 = x_29; +x_6 = x_30; +x_13 = x_27; +goto _start; } else { -lean_object* x_63; lean_object* x_64; lean_object* x_65; uint8_t x_66; -x_63 = lean_unsigned_to_nat(0u); -x_64 = l_Lean_Syntax_getArg(x_10, x_63); +uint8_t x_32; +lean_dec(x_12); +lean_dec(x_11); lean_dec(x_10); -x_65 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__5___closed__2; -lean_inc(x_64); -x_66 = l_Lean_Syntax_isOfKind(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; lean_object* x_78; lean_object* x_79; uint8_t x_80; lean_object* x_81; lean_object* x_82; uint8_t x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; uint8_t x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; uint8_t x_94; -lean_dec(x_64); -lean_dec(x_5); -x_67 = l_Lean_Elab_Command_getRef(x_6, x_7, x_8); -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 = l_Lean_replaceRef(x_1, x_68); -lean_dec(x_68); -x_71 = lean_ctor_get(x_6, 0); -lean_inc(x_71); -x_72 = lean_ctor_get(x_6, 1); -lean_inc(x_72); -x_73 = lean_ctor_get(x_6, 2); -lean_inc(x_73); -x_74 = lean_ctor_get(x_6, 3); -lean_inc(x_74); -x_75 = lean_ctor_get(x_6, 4); -lean_inc(x_75); -x_76 = lean_ctor_get(x_6, 5); -lean_inc(x_76); -x_77 = lean_ctor_get(x_6, 7); -lean_inc(x_77); -x_78 = lean_ctor_get(x_6, 8); -lean_inc(x_78); -x_79 = lean_ctor_get(x_6, 9); -lean_inc(x_79); -x_80 = lean_ctor_get_uint8(x_6, sizeof(void*)*10); -x_81 = lean_alloc_ctor(0, 10, 1); -lean_ctor_set(x_81, 0, x_71); -lean_ctor_set(x_81, 1, x_72); -lean_ctor_set(x_81, 2, x_73); -lean_ctor_set(x_81, 3, x_74); -lean_ctor_set(x_81, 4, x_75); -lean_ctor_set(x_81, 5, x_76); -lean_ctor_set(x_81, 6, x_70); -lean_ctor_set(x_81, 7, x_77); -lean_ctor_set(x_81, 8, x_78); -lean_ctor_set(x_81, 9, x_79); -lean_ctor_set_uint8(x_81, sizeof(void*)*10, x_80); -x_82 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__3; -x_83 = 2; -x_84 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_82, x_83, x_81, x_7, x_69); -x_85 = lean_ctor_get(x_84, 1); -lean_inc(x_85); -lean_dec(x_84); -x_86 = l_Lean_Elab_Command_getRef(x_6, x_7, x_85); -x_87 = lean_ctor_get(x_86, 0); -lean_inc(x_87); -x_88 = lean_ctor_get(x_86, 1); -lean_inc(x_88); -lean_dec(x_86); -x_89 = 0; -x_90 = l_Lean_SourceInfo_fromRef(x_87, x_89); -lean_dec(x_87); -x_91 = l_Lean_Elab_Command_getCurrMacroScope(x_6, x_7, x_88); -x_92 = lean_ctor_get(x_91, 1); -lean_inc(x_92); -lean_dec(x_91); -x_93 = l_Lean_Elab_Command_getMainModule___rarg(x_7, x_92); -x_94 = !lean_is_exclusive(x_93); -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_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; -x_95 = lean_ctor_get(x_93, 1); -x_96 = lean_ctor_get(x_93, 0); -lean_dec(x_96); -x_97 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__12; -x_98 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; -lean_inc(x_90); -x_99 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_99, 0, x_90); -lean_ctor_set(x_99, 1, x_97); -lean_ctor_set(x_99, 2, x_98); -x_100 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; -lean_inc(x_90); -lean_ctor_set_tag(x_93, 2); -lean_ctor_set(x_93, 1, x_100); -lean_ctor_set(x_93, 0, x_90); -x_101 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; -lean_inc(x_90); -x_102 = l_Lean_Syntax_node1(x_90, x_101, x_93); -lean_inc(x_90); -x_103 = l_Lean_Syntax_node1(x_90, x_97, x_102); -lean_inc_n(x_99, 4); -x_104 = l_Lean_Syntax_node6(x_90, x_2, x_99, x_99, x_99, x_103, x_99, x_99); -x_105 = lean_apply_4(x_3, x_104, x_6, x_7, x_95); -return x_105; -} -else +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_2); +lean_dec(x_1); +x_32 = !lean_is_exclusive(x_26); +if (x_32 == 0) { -lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; -x_106 = lean_ctor_get(x_93, 1); -lean_inc(x_106); -lean_dec(x_93); -x_107 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__12; -x_108 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; -lean_inc(x_90); -x_109 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_109, 0, x_90); -lean_ctor_set(x_109, 1, x_107); -lean_ctor_set(x_109, 2, x_108); -x_110 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; -lean_inc(x_90); -x_111 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_111, 0, x_90); -lean_ctor_set(x_111, 1, x_110); -x_112 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; -lean_inc(x_90); -x_113 = l_Lean_Syntax_node1(x_90, x_112, x_111); -lean_inc(x_90); -x_114 = l_Lean_Syntax_node1(x_90, x_107, x_113); -lean_inc_n(x_109, 4); -x_115 = l_Lean_Syntax_node6(x_90, x_2, x_109, x_109, x_109, x_114, x_109, x_109); -x_116 = lean_apply_4(x_3, x_115, x_6, x_7, x_106); -return x_116; -} +return x_26; } else { -lean_object* x_117; lean_object* x_118; lean_object* x_119; -x_117 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_117, 0, x_64); -x_118 = lean_box(0); -x_119 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__4(x_1, x_2, x_3, x_5, x_118, x_117, x_6, x_7, x_8); -return x_119; +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_26, 0); +x_34 = lean_ctor_get(x_26, 1); +lean_inc(x_34); +lean_inc(x_33); +lean_dec(x_26); +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +return x_35; } } } else { -lean_object* x_120; lean_object* x_121; lean_object* x_122; +uint8_t x_36; +lean_dec(x_16); +lean_dec(x_12); +lean_dec(x_11); lean_dec(x_10); -x_120 = lean_box(0); -x_121 = lean_box(0); -x_122 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__4(x_1, x_2, x_3, x_5, x_121, x_120, x_6, x_7, x_8); -return x_122; -} -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___closed__1() { -_start: +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_2); +lean_dec(x_1); +x_36 = !lean_is_exclusive(x_18); +if (x_36 == 0) { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("declModifiers", 13, 13); -return x_1; -} +return x_18; } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___closed__2() { -_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_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__1; -x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__7; -x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___closed__1; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; -} +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_18, 0); +x_38 = lean_ctor_get(x_18, 1); +lean_inc(x_38); +lean_inc(x_37); +lean_dec(x_18); +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; } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("docComment", 10, 10); -return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__1; -x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__7; -x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___closed__3; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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_9; -x_9 = lean_usize_dec_lt(x_4, x_3); -if (x_9 == 0) +uint8_t x_12; +x_12 = lean_usize_dec_lt(x_3, x_2); +if (x_12 == 0) { -lean_object* x_10; +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_1); -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_5); -lean_ctor_set(x_10, 1, x_8); -return x_10; +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_11; lean_object* x_12; lean_object* x_13; 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; uint8_t x_27; -x_11 = lean_array_uget(x_2, x_4); -x_19 = lean_ctor_get(x_11, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_11, 1); -lean_inc(x_20); -x_21 = lean_ctor_get(x_11, 2); -lean_inc(x_21); -x_22 = lean_ctor_get(x_11, 3); -lean_inc(x_22); -x_23 = lean_ctor_get(x_11, 4); -lean_inc(x_23); -lean_dec(x_11); -lean_inc(x_23); -lean_inc(x_22); -lean_inc(x_21); -lean_inc(x_1); +lean_object* x_14; lean_object* x_15; lean_object* x_16; +lean_dec(x_4); +x_14 = lean_array_uget(x_1, x_3); +x_15 = lean_ctor_get(x_14, 4); +lean_inc(x_15); +lean_inc(x_5); +lean_inc(x_15); +x_16 = l_Lean_mkConstWithLevelParams___at_Lean_Elab_Term_expandDeclId___spec__7(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; uint8_t x_24; lean_object* x_25; +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +x_19 = lean_ctor_get(x_14, 0); lean_inc(x_19); -x_24 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___boxed), 9, 5); -lean_closure_set(x_24, 0, x_19); -lean_closure_set(x_24, 1, x_1); -lean_closure_set(x_24, 2, x_21); -lean_closure_set(x_24, 3, x_22); -lean_closure_set(x_24, 4, x_23); -x_25 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___closed__2; -lean_inc(x_20); -x_26 = l_Lean_Syntax_isOfKind(x_20, x_25); -if (x_26 == 0) +x_20 = lean_unsigned_to_nat(1u); +x_21 = l_Lean_Syntax_getArg(x_19, x_20); +lean_dec(x_19); +x_22 = lean_box(0); +x_23 = lean_box(0); +x_24 = 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_25 = l_Lean_Elab_Term_addTermInfo_x27(x_21, x_17, x_22, x_22, x_23, x_24, x_5, x_6, x_7, x_8, x_9, x_10, x_18); +if (lean_obj_tag(x_25) == 0) { -uint8_t x_217; -x_217 = 0; -x_27 = x_217; -goto block_216; +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_26 = lean_ctor_get(x_25, 1); +lean_inc(x_26); +lean_dec(x_25); +x_27 = lean_ctor_get(x_14, 8); +lean_inc(x_27); +x_28 = lean_array_size(x_27); +x_29 = 0; +x_30 = 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_31 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__2(x_22, x_22, x_27, x_28, x_29, x_30, x_5, x_6, x_7, x_8, x_9, x_10, x_26); +lean_dec(x_27); +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; +x_32 = lean_ctor_get(x_31, 1); +lean_inc(x_32); +lean_dec(x_31); +x_33 = lean_ctor_get(x_14, 2); +lean_inc(x_33); +lean_dec(x_14); +x_34 = lean_ctor_get(x_33, 2); +lean_inc(x_34); +lean_dec(x_33); +x_35 = 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_36 = l_Lean_Elab_Term_applyAttributesAt(x_15, x_34, x_35, x_5, x_6, x_7, x_8, x_9, x_10, x_32); +if (lean_obj_tag(x_36) == 0) +{ +lean_object* x_37; size_t x_38; size_t x_39; +x_37 = lean_ctor_get(x_36, 1); +lean_inc(x_37); +lean_dec(x_36); +x_38 = 1; +x_39 = lean_usize_add(x_3, x_38); +x_3 = x_39; +x_4 = x_30; +x_11 = x_37; +goto _start; } else { -uint8_t x_218; -x_218 = 1; -x_27 = x_218; -goto block_216; +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_36); +if (x_41 == 0) +{ +return x_36; } -block_18: +else { -lean_object* x_14; size_t x_15; size_t x_16; -x_14 = lean_array_push(x_5, x_12); -x_15 = 1; -x_16 = lean_usize_add(x_4, x_15); -x_4 = x_16; -x_5 = x_14; -x_8 = x_13; -goto _start; +lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_42 = lean_ctor_get(x_36, 0); +x_43 = lean_ctor_get(x_36, 1); +lean_inc(x_43); +lean_inc(x_42); +lean_dec(x_36); +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; } -block_216: +} +} +else { -if (x_27 == 0) +uint8_t x_45; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_45 = !lean_is_exclusive(x_31); +if (x_45 == 0) { -lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; uint8_t 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_24); -x_28 = l_Lean_Elab_Command_getRef(x_6, x_7, x_8); -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_replaceRef(x_20, x_29); -lean_dec(x_29); -lean_dec(x_20); -x_32 = lean_ctor_get(x_6, 0); -lean_inc(x_32); -x_33 = lean_ctor_get(x_6, 1); -lean_inc(x_33); -x_34 = lean_ctor_get(x_6, 2); -lean_inc(x_34); -x_35 = lean_ctor_get(x_6, 3); -lean_inc(x_35); -x_36 = lean_ctor_get(x_6, 4); -lean_inc(x_36); -x_37 = lean_ctor_get(x_6, 5); -lean_inc(x_37); -x_38 = lean_ctor_get(x_6, 7); -lean_inc(x_38); -x_39 = lean_ctor_get(x_6, 8); -lean_inc(x_39); -x_40 = lean_ctor_get(x_6, 9); -lean_inc(x_40); -x_41 = lean_ctor_get_uint8(x_6, sizeof(void*)*10); -x_42 = lean_alloc_ctor(0, 10, 1); -lean_ctor_set(x_42, 0, x_32); -lean_ctor_set(x_42, 1, x_33); -lean_ctor_set(x_42, 2, x_34); -lean_ctor_set(x_42, 3, x_35); -lean_ctor_set(x_42, 4, x_36); -lean_ctor_set(x_42, 5, x_37); -lean_ctor_set(x_42, 6, x_31); -lean_ctor_set(x_42, 7, x_38); -lean_ctor_set(x_42, 8, x_39); -lean_ctor_set(x_42, 9, x_40); -lean_ctor_set_uint8(x_42, sizeof(void*)*10, x_41); -x_43 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__3; -x_44 = 2; -x_45 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_43, x_44, x_42, x_7, x_30); -x_46 = lean_ctor_get(x_45, 1); +return x_31; +} +else +{ +lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_46 = lean_ctor_get(x_31, 0); +x_47 = lean_ctor_get(x_31, 1); +lean_inc(x_47); lean_inc(x_46); -lean_dec(x_45); -x_47 = l_Lean_Elab_Command_getRef(x_6, x_7, x_46); -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 = 0; -x_51 = l_Lean_SourceInfo_fromRef(x_48, x_50); -lean_dec(x_48); -x_52 = l_Lean_Elab_Command_getCurrMacroScope(x_6, x_7, x_49); -x_53 = lean_ctor_get(x_52, 1); -lean_inc(x_53); -lean_dec(x_52); -x_54 = l_Lean_Elab_Command_getMainModule___rarg(x_7, x_53); -x_55 = !lean_is_exclusive(x_54); -if (x_55 == 0) +lean_dec(x_31); +x_48 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_48, 0, x_46); +lean_ctor_set(x_48, 1, x_47); +return x_48; +} +} +} +else { -lean_object* x_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_56 = lean_ctor_get(x_54, 1); -x_57 = lean_ctor_get(x_54, 0); -lean_dec(x_57); -x_58 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__12; -x_59 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; -lean_inc(x_51); -x_60 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_60, 0, x_51); -lean_ctor_set(x_60, 1, x_58); -lean_ctor_set(x_60, 2, x_59); -x_61 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; -lean_inc(x_51); -lean_ctor_set_tag(x_54, 2); -lean_ctor_set(x_54, 1, x_61); -lean_ctor_set(x_54, 0, x_51); -x_62 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; -lean_inc(x_51); -x_63 = l_Lean_Syntax_node1(x_51, x_62, x_54); +uint8_t x_49; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_49 = !lean_is_exclusive(x_25); +if (x_49 == 0) +{ +return x_25; +} +else +{ +lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_50 = lean_ctor_get(x_25, 0); +x_51 = lean_ctor_get(x_25, 1); lean_inc(x_51); -x_64 = l_Lean_Syntax_node1(x_51, x_58, x_63); -lean_inc_n(x_60, 4); -x_65 = l_Lean_Syntax_node6(x_51, x_25, x_60, x_60, x_60, x_64, x_60, x_60); +lean_inc(x_50); +lean_dec(x_25); +x_52 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_52, 0, x_50); +lean_ctor_set(x_52, 1, x_51); +return x_52; +} +} +} +else +{ +uint8_t x_53; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_53 = !lean_is_exclusive(x_16); +if (x_53 == 0) +{ +return x_16; +} +else +{ +lean_object* x_54; lean_object* x_55; lean_object* x_56; +x_54 = lean_ctor_get(x_16, 0); +x_55 = lean_ctor_get(x_16, 1); +lean_inc(x_55); +lean_inc(x_54); +lean_dec(x_16); +x_56 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_56, 0, x_54); +lean_ctor_set(x_56, 1, x_55); +return x_56; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__8(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_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; +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_7); +lean_inc(x_6); +lean_inc(x_2); lean_inc(x_1); -x_66 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1(x_19, x_1, x_21, x_22, x_23, x_65, x_6, x_7, x_56); +x_18 = l_Lean_PersistentArray_mapMAux___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__7(x_1, x_2, x_15, 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; 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_4, x_21); +x_23 = lean_array_uset(x_17, x_4, x_19); +x_4 = x_22; +x_5 = x_23; +x_12 = x_20; +goto _start; +} +else +{ +uint8_t x_25; +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_2); +lean_dec(x_1); +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_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__9(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_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; +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); +x_18 = lean_ctor_get(x_2, 0); +lean_inc(x_18); +x_19 = l_Lean_Elab_InfoTree_substitute(x_15, x_18); +lean_inc(x_1); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +x_20 = lean_apply_7(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_20) == 0) +{ +lean_object* x_21; +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +if (lean_obj_tag(x_21) == 0) +{ +lean_object* x_22; size_t x_23; size_t x_24; lean_object* x_25; +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +x_23 = 1; +x_24 = lean_usize_add(x_4, x_23); +x_25 = lean_array_uset(x_17, x_4, x_19); +x_4 = x_24; +x_5 = x_25; +x_12 = x_22; +goto _start; +} +else +{ +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_20, 1); +lean_inc(x_27); +lean_dec(x_20); +x_28 = lean_ctor_get(x_21, 0); +lean_inc(x_28); +lean_dec(x_21); +x_29 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_19); +x_30 = 1; +x_31 = lean_usize_add(x_4, x_30); +x_32 = lean_array_uset(x_17, x_4, x_29); +x_4 = x_31; +x_5 = x_32; +x_12 = x_27; +goto _start; +} +} +else +{ +uint8_t x_34; lean_dec(x_19); -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_12 = x_67; -x_13 = x_68; -goto block_18; +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_2); +lean_dec(x_1); +x_34 = !lean_is_exclusive(x_20); +if (x_34 == 0) +{ +return x_20; +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; +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_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +return x_37; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapMAux___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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: +{ +if (lean_obj_tag(x_3) == 0) +{ +uint8_t x_11; +x_11 = !lean_is_exclusive(x_3); +if (x_11 == 0) +{ +lean_object* x_12; size_t x_13; size_t x_14; lean_object* x_15; +x_12 = lean_ctor_get(x_3, 0); +x_13 = lean_array_size(x_12); +x_14 = 0; +x_15 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__8(x_1, x_2, x_13, x_14, x_12, 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; +x_16 = !lean_is_exclusive(x_15); +if (x_16 == 0) +{ +lean_object* x_17; +x_17 = lean_ctor_get(x_15, 0); +lean_ctor_set(x_3, 0, x_17); +lean_ctor_set(x_15, 0, x_3); +return x_15; +} +else +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_15, 0); +x_19 = lean_ctor_get(x_15, 1); +lean_inc(x_19); +lean_inc(x_18); +lean_dec(x_15); +lean_ctor_set(x_3, 0, x_18); +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_3); +lean_ctor_set(x_20, 1, x_19); +return x_20; +} +} +else +{ +uint8_t x_21; +lean_free_object(x_3); +x_21 = !lean_is_exclusive(x_15); +if (x_21 == 0) +{ +return x_15; +} +else +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_15, 0); +x_23 = lean_ctor_get(x_15, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_15); +x_24 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); +return x_24; +} +} +} +else +{ +lean_object* x_25; size_t x_26; size_t x_27; lean_object* x_28; +x_25 = lean_ctor_get(x_3, 0); +lean_inc(x_25); +lean_dec(x_3); +x_26 = lean_array_size(x_25); +x_27 = 0; +x_28 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__8(x_1, x_2, x_26, x_27, x_25, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_28) == 0) +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_29 = lean_ctor_get(x_28, 0); +lean_inc(x_29); +x_30 = lean_ctor_get(x_28, 1); +lean_inc(x_30); +if (lean_is_exclusive(x_28)) { + lean_ctor_release(x_28, 0); + lean_ctor_release(x_28, 1); + x_31 = x_28; +} else { + lean_dec_ref(x_28); + x_31 = lean_box(0); +} +x_32 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_32, 0, x_29); +if (lean_is_scalar(x_31)) { + x_33 = lean_alloc_ctor(0, 2, 0); +} else { + x_33 = x_31; +} +lean_ctor_set(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; +x_34 = lean_ctor_get(x_28, 0); +lean_inc(x_34); +x_35 = lean_ctor_get(x_28, 1); +lean_inc(x_35); +if (lean_is_exclusive(x_28)) { + lean_ctor_release(x_28, 0); + lean_ctor_release(x_28, 1); + x_36 = x_28; +} else { + lean_dec_ref(x_28); + x_36 = lean_box(0); +} +if (lean_is_scalar(x_36)) { + x_37 = lean_alloc_ctor(1, 2, 0); +} else { + x_37 = x_36; +} +lean_ctor_set(x_37, 0, x_34); +lean_ctor_set(x_37, 1, x_35); +return x_37; +} +} +} +else +{ +uint8_t x_38; +x_38 = !lean_is_exclusive(x_3); +if (x_38 == 0) +{ +lean_object* x_39; size_t x_40; size_t x_41; lean_object* x_42; +x_39 = lean_ctor_get(x_3, 0); +x_40 = lean_array_size(x_39); +x_41 = 0; +x_42 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__9(x_1, x_2, x_40, x_41, x_39, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_42) == 0) +{ +uint8_t x_43; +x_43 = !lean_is_exclusive(x_42); +if (x_43 == 0) +{ +lean_object* x_44; +x_44 = lean_ctor_get(x_42, 0); +lean_ctor_set(x_3, 0, x_44); +lean_ctor_set(x_42, 0, x_3); +return x_42; +} +else +{ +lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_45 = lean_ctor_get(x_42, 0); +x_46 = lean_ctor_get(x_42, 1); +lean_inc(x_46); +lean_inc(x_45); +lean_dec(x_42); +lean_ctor_set(x_3, 0, x_45); +x_47 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_47, 0, x_3); +lean_ctor_set(x_47, 1, x_46); +return x_47; +} +} +else +{ +uint8_t x_48; +lean_free_object(x_3); +x_48 = !lean_is_exclusive(x_42); +if (x_48 == 0) +{ +return x_42; +} +else +{ +lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_49 = lean_ctor_get(x_42, 0); +x_50 = lean_ctor_get(x_42, 1); +lean_inc(x_50); +lean_inc(x_49); +lean_dec(x_42); +x_51 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_51, 0, x_49); +lean_ctor_set(x_51, 1, x_50); +return x_51; +} +} +} +else +{ +lean_object* x_52; size_t x_53; size_t x_54; lean_object* x_55; +x_52 = lean_ctor_get(x_3, 0); +lean_inc(x_52); +lean_dec(x_3); +x_53 = lean_array_size(x_52); +x_54 = 0; +x_55 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__9(x_1, x_2, x_53, x_54, x_52, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_55) == 0) +{ +lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; +x_56 = lean_ctor_get(x_55, 0); +lean_inc(x_56); +x_57 = lean_ctor_get(x_55, 1); +lean_inc(x_57); +if (lean_is_exclusive(x_55)) { + lean_ctor_release(x_55, 0); + lean_ctor_release(x_55, 1); + x_58 = x_55; +} else { + lean_dec_ref(x_55); + x_58 = lean_box(0); +} +x_59 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_59, 0, x_56); +if (lean_is_scalar(x_58)) { + x_60 = lean_alloc_ctor(0, 2, 0); +} else { + x_60 = x_58; +} +lean_ctor_set(x_60, 0, x_59); +lean_ctor_set(x_60, 1, x_57); +return x_60; +} +else +{ +lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; +x_61 = lean_ctor_get(x_55, 0); +lean_inc(x_61); +x_62 = lean_ctor_get(x_55, 1); +lean_inc(x_62); +if (lean_is_exclusive(x_55)) { + lean_ctor_release(x_55, 0); + lean_ctor_release(x_55, 1); + x_63 = x_55; +} else { + lean_dec_ref(x_55); + x_63 = lean_box(0); +} +if (lean_is_scalar(x_63)) { + x_64 = lean_alloc_ctor(1, 2, 0); +} else { + x_64 = x_63; +} +lean_ctor_set(x_64, 0, x_61); +lean_ctor_set(x_64, 1, x_62); +return x_64; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__10(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_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; +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); +x_18 = lean_ctor_get(x_2, 0); +lean_inc(x_18); +x_19 = l_Lean_Elab_InfoTree_substitute(x_15, x_18); +lean_inc(x_1); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +x_20 = lean_apply_7(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_20) == 0) +{ +lean_object* x_21; +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +if (lean_obj_tag(x_21) == 0) +{ +lean_object* x_22; size_t x_23; size_t x_24; lean_object* x_25; +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +x_23 = 1; +x_24 = lean_usize_add(x_4, x_23); +x_25 = lean_array_uset(x_17, x_4, x_19); +x_4 = x_24; +x_5 = x_25; +x_12 = x_22; +goto _start; +} +else +{ +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_20, 1); +lean_inc(x_27); +lean_dec(x_20); +x_28 = lean_ctor_get(x_21, 0); +lean_inc(x_28); +lean_dec(x_21); +x_29 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_19); +x_30 = 1; +x_31 = lean_usize_add(x_4, x_30); +x_32 = lean_array_uset(x_17, x_4, x_29); +x_4 = x_31; +x_5 = x_32; +x_12 = x_27; +goto _start; +} +} +else +{ +uint8_t x_34; +lean_dec(x_19); +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_2); +lean_dec(x_1); +x_34 = !lean_is_exclusive(x_20); +if (x_34 == 0) +{ +return x_20; +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; +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_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +return x_37; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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: +{ +uint8_t x_11; +x_11 = !lean_is_exclusive(x_3); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_12 = lean_ctor_get(x_3, 0); +x_13 = lean_ctor_get(x_3, 1); +x_14 = lean_ctor_get(x_3, 2); +x_15 = lean_ctor_get(x_3, 3); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_2); +lean_inc(x_1); +x_16 = l_Lean_PersistentArray_mapMAux___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__7(x_1, x_2, x_12, x_4, x_5, 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; size_t x_19; size_t x_20; lean_object* x_21; +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +x_19 = lean_array_size(x_13); +x_20 = 0; +x_21 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__10(x_1, x_2, x_19, x_20, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_18); +if (lean_obj_tag(x_21) == 0) +{ +uint8_t x_22; +x_22 = !lean_is_exclusive(x_21); +if (x_22 == 0) +{ +lean_object* x_23; +x_23 = lean_ctor_get(x_21, 0); +lean_ctor_set(x_3, 1, x_23); +lean_ctor_set(x_3, 0, x_17); +lean_ctor_set(x_21, 0, x_3); +return x_21; +} +else +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_21, 0); +x_25 = lean_ctor_get(x_21, 1); +lean_inc(x_25); +lean_inc(x_24); +lean_dec(x_21); +lean_ctor_set(x_3, 1, x_24); +lean_ctor_set(x_3, 0, x_17); +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_3); +lean_ctor_set(x_26, 1, x_25); +return x_26; +} +} +else +{ +uint8_t x_27; +lean_dec(x_17); +lean_free_object(x_3); +lean_dec(x_15); +lean_dec(x_14); +x_27 = !lean_is_exclusive(x_21); +if (x_27 == 0) +{ +return x_21; +} +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; +} +} +} +else +{ +uint8_t x_31; +lean_free_object(x_3); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +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; +} +} +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; size_t x_38; lean_object* x_39; lean_object* x_40; +x_35 = lean_ctor_get(x_3, 0); +x_36 = lean_ctor_get(x_3, 1); +x_37 = lean_ctor_get(x_3, 2); +x_38 = lean_ctor_get_usize(x_3, 4); +x_39 = lean_ctor_get(x_3, 3); +lean_inc(x_39); +lean_inc(x_37); +lean_inc(x_36); +lean_inc(x_35); +lean_dec(x_3); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_2); +lean_inc(x_1); +x_40 = l_Lean_PersistentArray_mapMAux___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__7(x_1, x_2, x_35, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_40) == 0) +{ +lean_object* x_41; lean_object* x_42; size_t x_43; size_t x_44; lean_object* x_45; +x_41 = lean_ctor_get(x_40, 0); +lean_inc(x_41); +x_42 = lean_ctor_get(x_40, 1); +lean_inc(x_42); +lean_dec(x_40); +x_43 = lean_array_size(x_36); +x_44 = 0; +x_45 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__10(x_1, x_2, x_43, x_44, x_36, x_4, x_5, x_6, x_7, x_8, x_9, x_42); +if (lean_obj_tag(x_45) == 0) +{ +lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_46 = lean_ctor_get(x_45, 0); +lean_inc(x_46); +x_47 = lean_ctor_get(x_45, 1); +lean_inc(x_47); +if (lean_is_exclusive(x_45)) { + lean_ctor_release(x_45, 0); + lean_ctor_release(x_45, 1); + x_48 = x_45; +} else { + lean_dec_ref(x_45); + x_48 = lean_box(0); +} +x_49 = lean_alloc_ctor(0, 4, sizeof(size_t)*1); +lean_ctor_set(x_49, 0, x_41); +lean_ctor_set(x_49, 1, x_46); +lean_ctor_set(x_49, 2, x_37); +lean_ctor_set(x_49, 3, x_39); +lean_ctor_set_usize(x_49, 4, x_38); +if (lean_is_scalar(x_48)) { + x_50 = lean_alloc_ctor(0, 2, 0); +} else { + x_50 = x_48; +} +lean_ctor_set(x_50, 0, x_49); +lean_ctor_set(x_50, 1, x_47); +return x_50; +} +else +{ +lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +lean_dec(x_41); +lean_dec(x_39); +lean_dec(x_37); +x_51 = lean_ctor_get(x_45, 0); +lean_inc(x_51); +x_52 = lean_ctor_get(x_45, 1); +lean_inc(x_52); +if (lean_is_exclusive(x_45)) { + lean_ctor_release(x_45, 0); + lean_ctor_release(x_45, 1); + x_53 = x_45; +} else { + lean_dec_ref(x_45); + x_53 = lean_box(0); +} +if (lean_is_scalar(x_53)) { + x_54 = lean_alloc_ctor(1, 2, 0); +} else { + x_54 = x_53; +} +lean_ctor_set(x_54, 0, x_51); +lean_ctor_set(x_54, 1, x_52); +return x_54; +} +} +else +{ +lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; +lean_dec(x_39); +lean_dec(x_37); +lean_dec(x_36); +lean_dec(x_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_55 = lean_ctor_get(x_40, 0); +lean_inc(x_55); +x_56 = lean_ctor_get(x_40, 1); +lean_inc(x_56); +if (lean_is_exclusive(x_40)) { + lean_ctor_release(x_40, 0); + lean_ctor_release(x_40, 1); + x_57 = x_40; +} else { + lean_dec_ref(x_40); + 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_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__13(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_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; +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_7); +lean_inc(x_6); +lean_inc(x_2); +lean_inc(x_1); +x_18 = l_Lean_PersistentArray_mapMAux___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__12(x_1, x_2, x_15, 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; 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_4, x_21); +x_23 = lean_array_uset(x_17, x_4, x_19); +x_4 = x_22; +x_5 = x_23; +x_12 = x_20; +goto _start; +} +else +{ +uint8_t x_25; +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_2); +lean_dec(x_1); +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_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__14(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_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; +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); +x_18 = lean_ctor_get(x_2, 0); +lean_inc(x_18); +x_19 = l_Lean_Elab_InfoTree_substitute(x_15, x_18); +lean_inc(x_1); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +x_20 = lean_apply_7(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_20) == 0) +{ +lean_object* x_21; +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +if (lean_obj_tag(x_21) == 0) +{ +lean_object* x_22; size_t x_23; size_t x_24; lean_object* x_25; +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +x_23 = 1; +x_24 = lean_usize_add(x_4, x_23); +x_25 = lean_array_uset(x_17, x_4, x_19); +x_4 = x_24; +x_5 = x_25; +x_12 = x_22; +goto _start; +} +else +{ +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_20, 1); +lean_inc(x_27); +lean_dec(x_20); +x_28 = lean_ctor_get(x_21, 0); +lean_inc(x_28); +lean_dec(x_21); +x_29 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_19); +x_30 = 1; +x_31 = lean_usize_add(x_4, x_30); +x_32 = lean_array_uset(x_17, x_4, x_29); +x_4 = x_31; +x_5 = x_32; +x_12 = x_27; +goto _start; +} +} +else +{ +uint8_t x_34; +lean_dec(x_19); +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_2); +lean_dec(x_1); +x_34 = !lean_is_exclusive(x_20); +if (x_34 == 0) +{ +return x_20; +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; +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_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +return x_37; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapMAux___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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: +{ +if (lean_obj_tag(x_3) == 0) +{ +uint8_t x_11; +x_11 = !lean_is_exclusive(x_3); +if (x_11 == 0) +{ +lean_object* x_12; size_t x_13; size_t x_14; lean_object* x_15; +x_12 = lean_ctor_get(x_3, 0); +x_13 = lean_array_size(x_12); +x_14 = 0; +x_15 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__13(x_1, x_2, x_13, x_14, x_12, 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; +x_16 = !lean_is_exclusive(x_15); +if (x_16 == 0) +{ +lean_object* x_17; +x_17 = lean_ctor_get(x_15, 0); +lean_ctor_set(x_3, 0, x_17); +lean_ctor_set(x_15, 0, x_3); +return x_15; +} +else +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_15, 0); +x_19 = lean_ctor_get(x_15, 1); +lean_inc(x_19); +lean_inc(x_18); +lean_dec(x_15); +lean_ctor_set(x_3, 0, x_18); +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_3); +lean_ctor_set(x_20, 1, x_19); +return x_20; +} +} +else +{ +uint8_t x_21; +lean_free_object(x_3); +x_21 = !lean_is_exclusive(x_15); +if (x_21 == 0) +{ +return x_15; +} +else +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_15, 0); +x_23 = lean_ctor_get(x_15, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_15); +x_24 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); +return x_24; +} +} +} +else +{ +lean_object* x_25; size_t x_26; size_t x_27; lean_object* x_28; +x_25 = lean_ctor_get(x_3, 0); +lean_inc(x_25); +lean_dec(x_3); +x_26 = lean_array_size(x_25); +x_27 = 0; +x_28 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__13(x_1, x_2, x_26, x_27, x_25, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_28) == 0) +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_29 = lean_ctor_get(x_28, 0); +lean_inc(x_29); +x_30 = lean_ctor_get(x_28, 1); +lean_inc(x_30); +if (lean_is_exclusive(x_28)) { + lean_ctor_release(x_28, 0); + lean_ctor_release(x_28, 1); + x_31 = x_28; +} else { + lean_dec_ref(x_28); + x_31 = lean_box(0); +} +x_32 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_32, 0, x_29); +if (lean_is_scalar(x_31)) { + x_33 = lean_alloc_ctor(0, 2, 0); +} else { + x_33 = x_31; +} +lean_ctor_set(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; +x_34 = lean_ctor_get(x_28, 0); +lean_inc(x_34); +x_35 = lean_ctor_get(x_28, 1); +lean_inc(x_35); +if (lean_is_exclusive(x_28)) { + lean_ctor_release(x_28, 0); + lean_ctor_release(x_28, 1); + x_36 = x_28; +} else { + lean_dec_ref(x_28); + x_36 = lean_box(0); +} +if (lean_is_scalar(x_36)) { + x_37 = lean_alloc_ctor(1, 2, 0); +} else { + x_37 = x_36; +} +lean_ctor_set(x_37, 0, x_34); +lean_ctor_set(x_37, 1, x_35); +return x_37; +} +} +} +else +{ +uint8_t x_38; +x_38 = !lean_is_exclusive(x_3); +if (x_38 == 0) +{ +lean_object* x_39; size_t x_40; size_t x_41; lean_object* x_42; +x_39 = lean_ctor_get(x_3, 0); +x_40 = lean_array_size(x_39); +x_41 = 0; +x_42 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__14(x_1, x_2, x_40, x_41, x_39, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_42) == 0) +{ +uint8_t x_43; +x_43 = !lean_is_exclusive(x_42); +if (x_43 == 0) +{ +lean_object* x_44; +x_44 = lean_ctor_get(x_42, 0); +lean_ctor_set(x_3, 0, x_44); +lean_ctor_set(x_42, 0, x_3); +return x_42; +} +else +{ +lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_45 = lean_ctor_get(x_42, 0); +x_46 = lean_ctor_get(x_42, 1); +lean_inc(x_46); +lean_inc(x_45); +lean_dec(x_42); +lean_ctor_set(x_3, 0, x_45); +x_47 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_47, 0, x_3); +lean_ctor_set(x_47, 1, x_46); +return x_47; +} +} +else +{ +uint8_t x_48; +lean_free_object(x_3); +x_48 = !lean_is_exclusive(x_42); +if (x_48 == 0) +{ +return x_42; +} +else +{ +lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_49 = lean_ctor_get(x_42, 0); +x_50 = lean_ctor_get(x_42, 1); +lean_inc(x_50); +lean_inc(x_49); +lean_dec(x_42); +x_51 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_51, 0, x_49); +lean_ctor_set(x_51, 1, x_50); +return x_51; +} +} +} +else +{ +lean_object* x_52; size_t x_53; size_t x_54; lean_object* x_55; +x_52 = lean_ctor_get(x_3, 0); +lean_inc(x_52); +lean_dec(x_3); +x_53 = lean_array_size(x_52); +x_54 = 0; +x_55 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__14(x_1, x_2, x_53, x_54, x_52, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_55) == 0) +{ +lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; +x_56 = lean_ctor_get(x_55, 0); +lean_inc(x_56); +x_57 = lean_ctor_get(x_55, 1); +lean_inc(x_57); +if (lean_is_exclusive(x_55)) { + lean_ctor_release(x_55, 0); + lean_ctor_release(x_55, 1); + x_58 = x_55; +} else { + lean_dec_ref(x_55); + x_58 = lean_box(0); +} +x_59 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_59, 0, x_56); +if (lean_is_scalar(x_58)) { + x_60 = lean_alloc_ctor(0, 2, 0); +} else { + x_60 = x_58; +} +lean_ctor_set(x_60, 0, x_59); +lean_ctor_set(x_60, 1, x_57); +return x_60; +} +else +{ +lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; +x_61 = lean_ctor_get(x_55, 0); +lean_inc(x_61); +x_62 = lean_ctor_get(x_55, 1); +lean_inc(x_62); +if (lean_is_exclusive(x_55)) { + lean_ctor_release(x_55, 0); + lean_ctor_release(x_55, 1); + x_63 = x_55; +} else { + lean_dec_ref(x_55); + x_63 = lean_box(0); +} +if (lean_is_scalar(x_63)) { + x_64 = lean_alloc_ctor(1, 2, 0); +} else { + x_64 = x_63; +} +lean_ctor_set(x_64, 0, x_61); +lean_ctor_set(x_64, 1, x_62); +return x_64; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__15(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_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; +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); +x_18 = lean_ctor_get(x_2, 0); +lean_inc(x_18); +x_19 = l_Lean_Elab_InfoTree_substitute(x_15, x_18); +lean_inc(x_1); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +x_20 = lean_apply_7(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_20) == 0) +{ +lean_object* x_21; +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +if (lean_obj_tag(x_21) == 0) +{ +lean_object* x_22; size_t x_23; size_t x_24; lean_object* x_25; +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +x_23 = 1; +x_24 = lean_usize_add(x_4, x_23); +x_25 = lean_array_uset(x_17, x_4, x_19); +x_4 = x_24; +x_5 = x_25; +x_12 = x_22; +goto _start; +} +else +{ +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_20, 1); +lean_inc(x_27); +lean_dec(x_20); +x_28 = lean_ctor_get(x_21, 0); +lean_inc(x_28); +lean_dec(x_21); +x_29 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_19); +x_30 = 1; +x_31 = lean_usize_add(x_4, x_30); +x_32 = lean_array_uset(x_17, x_4, x_29); +x_4 = x_31; +x_5 = x_32; +x_12 = x_27; +goto _start; +} +} +else +{ +uint8_t x_34; +lean_dec(x_19); +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_2); +lean_dec(x_1); +x_34 = !lean_is_exclusive(x_20); +if (x_34 == 0) +{ +return x_20; +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; +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_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +return x_37; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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: +{ +uint8_t x_11; +x_11 = !lean_is_exclusive(x_3); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_12 = lean_ctor_get(x_3, 0); +x_13 = lean_ctor_get(x_3, 1); +x_14 = lean_ctor_get(x_3, 2); +x_15 = lean_ctor_get(x_3, 3); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_2); +lean_inc(x_1); +x_16 = l_Lean_PersistentArray_mapMAux___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__12(x_1, x_2, x_12, x_4, x_5, 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; size_t x_19; size_t x_20; lean_object* x_21; +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +x_19 = lean_array_size(x_13); +x_20 = 0; +x_21 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__15(x_1, x_2, x_19, x_20, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_18); +if (lean_obj_tag(x_21) == 0) +{ +uint8_t x_22; +x_22 = !lean_is_exclusive(x_21); +if (x_22 == 0) +{ +lean_object* x_23; +x_23 = lean_ctor_get(x_21, 0); +lean_ctor_set(x_3, 1, x_23); +lean_ctor_set(x_3, 0, x_17); +lean_ctor_set(x_21, 0, x_3); +return x_21; +} +else +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_21, 0); +x_25 = lean_ctor_get(x_21, 1); +lean_inc(x_25); +lean_inc(x_24); +lean_dec(x_21); +lean_ctor_set(x_3, 1, x_24); +lean_ctor_set(x_3, 0, x_17); +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_3); +lean_ctor_set(x_26, 1, x_25); +return x_26; +} +} +else +{ +uint8_t x_27; +lean_dec(x_17); +lean_free_object(x_3); +lean_dec(x_15); +lean_dec(x_14); +x_27 = !lean_is_exclusive(x_21); +if (x_27 == 0) +{ +return x_21; +} +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; +} +} +} +else +{ +uint8_t x_31; +lean_free_object(x_3); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +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; +} +} +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; size_t x_38; lean_object* x_39; lean_object* x_40; +x_35 = lean_ctor_get(x_3, 0); +x_36 = lean_ctor_get(x_3, 1); +x_37 = lean_ctor_get(x_3, 2); +x_38 = lean_ctor_get_usize(x_3, 4); +x_39 = lean_ctor_get(x_3, 3); +lean_inc(x_39); +lean_inc(x_37); +lean_inc(x_36); +lean_inc(x_35); +lean_dec(x_3); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_2); +lean_inc(x_1); +x_40 = l_Lean_PersistentArray_mapMAux___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__12(x_1, x_2, x_35, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_40) == 0) +{ +lean_object* x_41; lean_object* x_42; size_t x_43; size_t x_44; lean_object* x_45; +x_41 = lean_ctor_get(x_40, 0); +lean_inc(x_41); +x_42 = lean_ctor_get(x_40, 1); +lean_inc(x_42); +lean_dec(x_40); +x_43 = lean_array_size(x_36); +x_44 = 0; +x_45 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__15(x_1, x_2, x_43, x_44, x_36, x_4, x_5, x_6, x_7, x_8, x_9, x_42); +if (lean_obj_tag(x_45) == 0) +{ +lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_46 = lean_ctor_get(x_45, 0); +lean_inc(x_46); +x_47 = lean_ctor_get(x_45, 1); +lean_inc(x_47); +if (lean_is_exclusive(x_45)) { + lean_ctor_release(x_45, 0); + lean_ctor_release(x_45, 1); + x_48 = x_45; +} else { + lean_dec_ref(x_45); + x_48 = lean_box(0); +} +x_49 = lean_alloc_ctor(0, 4, sizeof(size_t)*1); +lean_ctor_set(x_49, 0, x_41); +lean_ctor_set(x_49, 1, x_46); +lean_ctor_set(x_49, 2, x_37); +lean_ctor_set(x_49, 3, x_39); +lean_ctor_set_usize(x_49, 4, x_38); +if (lean_is_scalar(x_48)) { + x_50 = lean_alloc_ctor(0, 2, 0); +} else { + x_50 = x_48; +} +lean_ctor_set(x_50, 0, x_49); +lean_ctor_set(x_50, 1, x_47); +return x_50; +} +else +{ +lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +lean_dec(x_41); +lean_dec(x_39); +lean_dec(x_37); +x_51 = lean_ctor_get(x_45, 0); +lean_inc(x_51); +x_52 = lean_ctor_get(x_45, 1); +lean_inc(x_52); +if (lean_is_exclusive(x_45)) { + lean_ctor_release(x_45, 0); + lean_ctor_release(x_45, 1); + x_53 = x_45; +} else { + lean_dec_ref(x_45); + x_53 = lean_box(0); +} +if (lean_is_scalar(x_53)) { + x_54 = lean_alloc_ctor(1, 2, 0); +} else { + x_54 = x_53; +} +lean_ctor_set(x_54, 0, x_51); +lean_ctor_set(x_54, 1, x_52); +return x_54; +} +} +else +{ +lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; +lean_dec(x_39); +lean_dec(x_37); +lean_dec(x_36); +lean_dec(x_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_55 = lean_ctor_get(x_40, 0); +lean_inc(x_55); +x_56 = lean_ctor_get(x_40, 1); +lean_inc(x_56); +if (lean_is_exclusive(x_40)) { + lean_ctor_release(x_40, 0); + lean_ctor_release(x_40, 1); + x_57 = x_40; +} else { + lean_dec_ref(x_40); + 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_EXPORT lean_object* l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__5___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_11 = l_Lean_Elab_getResetInfoTrees___at_Lean_Elab_Term_withDeclName___spec__3___rarg(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); +x_14 = lean_apply_7(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +if (lean_obj_tag(x_14) == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +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_9, x_16); +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); +lean_dec(x_17); +x_20 = lean_ctor_get(x_18, 6); +lean_inc(x_20); +lean_dec(x_18); +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_inc(x_9); +x_22 = l_Lean_PersistentArray_mapM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__6(x_2, x_20, x_21, x_4, x_5, x_6, x_7, x_8, x_9, x_19); +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; uint8_t x_29; +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_st_ref_take(x_9, x_24); +x_26 = lean_ctor_get(x_25, 0); +lean_inc(x_26); +x_27 = lean_ctor_get(x_26, 6); +lean_inc(x_27); +x_28 = lean_ctor_get(x_25, 1); +lean_inc(x_28); +lean_dec(x_25); +x_29 = !lean_is_exclusive(x_26); +if (x_29 == 0) +{ +lean_object* x_30; uint8_t x_31; +x_30 = lean_ctor_get(x_26, 6); +lean_dec(x_30); +x_31 = !lean_is_exclusive(x_27); +if (x_31 == 0) +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; +x_32 = lean_ctor_get(x_27, 1); +lean_dec(x_32); +x_33 = l_Lean_PersistentArray_append___rarg(x_12, x_23); +lean_dec(x_23); +lean_ctor_set(x_27, 1, x_33); +x_34 = lean_st_ref_set(x_9, x_26, x_28); +lean_dec(x_9); +x_35 = !lean_is_exclusive(x_34); +if (x_35 == 0) +{ +lean_object* x_36; +x_36 = lean_ctor_get(x_34, 0); +lean_dec(x_36); +lean_ctor_set(x_34, 0, x_15); +return x_34; +} +else +{ +lean_object* x_37; lean_object* x_38; +x_37 = lean_ctor_get(x_34, 1); +lean_inc(x_37); +lean_dec(x_34); +x_38 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_38, 0, x_15); +lean_ctor_set(x_38, 1, x_37); +return x_38; +} +} +else +{ +uint8_t x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_39 = lean_ctor_get_uint8(x_27, sizeof(void*)*2); +x_40 = lean_ctor_get(x_27, 0); +lean_inc(x_40); +lean_dec(x_27); +x_41 = l_Lean_PersistentArray_append___rarg(x_12, x_23); +lean_dec(x_23); +x_42 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_42, 0, x_40); +lean_ctor_set(x_42, 1, x_41); +lean_ctor_set_uint8(x_42, sizeof(void*)*2, x_39); +lean_ctor_set(x_26, 6, x_42); +x_43 = lean_st_ref_set(x_9, x_26, x_28); +lean_dec(x_9); +x_44 = lean_ctor_get(x_43, 1); +lean_inc(x_44); +if (lean_is_exclusive(x_43)) { + lean_ctor_release(x_43, 0); + lean_ctor_release(x_43, 1); + x_45 = x_43; +} else { + lean_dec_ref(x_43); + x_45 = lean_box(0); +} +if (lean_is_scalar(x_45)) { + x_46 = lean_alloc_ctor(0, 2, 0); +} else { + x_46 = x_45; +} +lean_ctor_set(x_46, 0, x_15); +lean_ctor_set(x_46, 1, x_44); +return x_46; +} +} +else +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; uint8_t x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; +x_47 = lean_ctor_get(x_26, 0); +x_48 = lean_ctor_get(x_26, 1); +x_49 = lean_ctor_get(x_26, 2); +x_50 = lean_ctor_get(x_26, 3); +x_51 = lean_ctor_get(x_26, 4); +x_52 = lean_ctor_get(x_26, 5); +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_dec(x_26); +x_53 = lean_ctor_get_uint8(x_27, sizeof(void*)*2); +x_54 = lean_ctor_get(x_27, 0); +lean_inc(x_54); +if (lean_is_exclusive(x_27)) { + lean_ctor_release(x_27, 0); + lean_ctor_release(x_27, 1); + x_55 = x_27; +} else { + lean_dec_ref(x_27); + x_55 = lean_box(0); +} +x_56 = l_Lean_PersistentArray_append___rarg(x_12, x_23); +lean_dec(x_23); +if (lean_is_scalar(x_55)) { + x_57 = lean_alloc_ctor(0, 2, 1); +} else { + x_57 = x_55; +} +lean_ctor_set(x_57, 0, x_54); +lean_ctor_set(x_57, 1, x_56); +lean_ctor_set_uint8(x_57, sizeof(void*)*2, x_53); +x_58 = lean_alloc_ctor(0, 7, 0); +lean_ctor_set(x_58, 0, x_47); +lean_ctor_set(x_58, 1, x_48); +lean_ctor_set(x_58, 2, x_49); +lean_ctor_set(x_58, 3, x_50); +lean_ctor_set(x_58, 4, x_51); +lean_ctor_set(x_58, 5, x_52); +lean_ctor_set(x_58, 6, x_57); +x_59 = lean_st_ref_set(x_9, x_58, x_28); +lean_dec(x_9); +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; +} else { + lean_dec_ref(x_59); + x_61 = lean_box(0); +} +if (lean_is_scalar(x_61)) { + x_62 = lean_alloc_ctor(0, 2, 0); +} else { + x_62 = x_61; +} +lean_ctor_set(x_62, 0, x_15); +lean_ctor_set(x_62, 1, x_60); +return x_62; +} +} +else +{ +uint8_t x_63; +lean_dec(x_15); +lean_dec(x_12); +lean_dec(x_9); +x_63 = !lean_is_exclusive(x_22); +if (x_63 == 0) +{ +return x_22; +} +else +{ +lean_object* x_64; lean_object* x_65; lean_object* x_66; +x_64 = lean_ctor_get(x_22, 0); +x_65 = lean_ctor_get(x_22, 1); +lean_inc(x_65); +lean_inc(x_64); +lean_dec(x_22); +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_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; +x_67 = lean_ctor_get(x_14, 0); +lean_inc(x_67); +x_68 = lean_ctor_get(x_14, 1); +lean_inc(x_68); +lean_dec(x_14); +x_69 = lean_st_ref_get(x_9, x_68); +x_70 = lean_ctor_get(x_69, 0); +lean_inc(x_70); +x_71 = lean_ctor_get(x_69, 1); +lean_inc(x_71); +lean_dec(x_69); +x_72 = lean_ctor_get(x_70, 6); +lean_inc(x_72); +lean_dec(x_70); +x_73 = lean_ctor_get(x_72, 1); +lean_inc(x_73); +lean_inc(x_9); +x_74 = l_Lean_PersistentArray_mapM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__11(x_2, x_72, x_73, x_4, x_5, x_6, x_7, x_8, x_9, x_71); +if (lean_obj_tag(x_74) == 0) +{ +lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; uint8_t x_81; +x_75 = lean_ctor_get(x_74, 0); +lean_inc(x_75); +x_76 = lean_ctor_get(x_74, 1); +lean_inc(x_76); +lean_dec(x_74); +x_77 = lean_st_ref_take(x_9, x_76); +x_78 = lean_ctor_get(x_77, 0); +lean_inc(x_78); +x_79 = lean_ctor_get(x_78, 6); +lean_inc(x_79); +x_80 = lean_ctor_get(x_77, 1); +lean_inc(x_80); +lean_dec(x_77); +x_81 = !lean_is_exclusive(x_78); +if (x_81 == 0) +{ +lean_object* x_82; uint8_t x_83; +x_82 = lean_ctor_get(x_78, 6); +lean_dec(x_82); +x_83 = !lean_is_exclusive(x_79); +if (x_83 == 0) +{ +lean_object* x_84; lean_object* x_85; lean_object* x_86; uint8_t x_87; +x_84 = lean_ctor_get(x_79, 1); +lean_dec(x_84); +x_85 = l_Lean_PersistentArray_append___rarg(x_12, x_75); +lean_dec(x_75); +lean_ctor_set(x_79, 1, x_85); +x_86 = lean_st_ref_set(x_9, x_78, x_80); +lean_dec(x_9); +x_87 = !lean_is_exclusive(x_86); +if (x_87 == 0) +{ +lean_object* x_88; +x_88 = lean_ctor_get(x_86, 0); +lean_dec(x_88); +lean_ctor_set_tag(x_86, 1); +lean_ctor_set(x_86, 0, x_67); +return x_86; +} +else +{ +lean_object* x_89; lean_object* x_90; +x_89 = lean_ctor_get(x_86, 1); +lean_inc(x_89); +lean_dec(x_86); +x_90 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_90, 0, x_67); +lean_ctor_set(x_90, 1, x_89); +return x_90; +} +} +else +{ +uint8_t x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; +x_91 = lean_ctor_get_uint8(x_79, sizeof(void*)*2); +x_92 = lean_ctor_get(x_79, 0); +lean_inc(x_92); +lean_dec(x_79); +x_93 = l_Lean_PersistentArray_append___rarg(x_12, x_75); +lean_dec(x_75); +x_94 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_94, 0, x_92); +lean_ctor_set(x_94, 1, x_93); +lean_ctor_set_uint8(x_94, sizeof(void*)*2, x_91); +lean_ctor_set(x_78, 6, x_94); +x_95 = lean_st_ref_set(x_9, x_78, x_80); +lean_dec(x_9); +x_96 = lean_ctor_get(x_95, 1); +lean_inc(x_96); +if (lean_is_exclusive(x_95)) { + lean_ctor_release(x_95, 0); + lean_ctor_release(x_95, 1); + x_97 = x_95; +} else { + lean_dec_ref(x_95); + x_97 = lean_box(0); +} +if (lean_is_scalar(x_97)) { + x_98 = lean_alloc_ctor(1, 2, 0); +} else { + x_98 = x_97; + lean_ctor_set_tag(x_98, 1); +} +lean_ctor_set(x_98, 0, x_67); +lean_ctor_set(x_98, 1, x_96); +return x_98; +} +} +else +{ +lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; 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; lean_object* x_113; lean_object* x_114; +x_99 = lean_ctor_get(x_78, 0); +x_100 = lean_ctor_get(x_78, 1); +x_101 = lean_ctor_get(x_78, 2); +x_102 = lean_ctor_get(x_78, 3); +x_103 = lean_ctor_get(x_78, 4); +x_104 = lean_ctor_get(x_78, 5); +lean_inc(x_104); +lean_inc(x_103); +lean_inc(x_102); +lean_inc(x_101); +lean_inc(x_100); +lean_inc(x_99); +lean_dec(x_78); +x_105 = lean_ctor_get_uint8(x_79, sizeof(void*)*2); +x_106 = lean_ctor_get(x_79, 0); +lean_inc(x_106); +if (lean_is_exclusive(x_79)) { + lean_ctor_release(x_79, 0); + lean_ctor_release(x_79, 1); + x_107 = x_79; +} else { + lean_dec_ref(x_79); + x_107 = lean_box(0); +} +x_108 = l_Lean_PersistentArray_append___rarg(x_12, x_75); +lean_dec(x_75); +if (lean_is_scalar(x_107)) { + x_109 = lean_alloc_ctor(0, 2, 1); +} else { + x_109 = x_107; +} +lean_ctor_set(x_109, 0, x_106); +lean_ctor_set(x_109, 1, x_108); +lean_ctor_set_uint8(x_109, sizeof(void*)*2, x_105); +x_110 = lean_alloc_ctor(0, 7, 0); +lean_ctor_set(x_110, 0, x_99); +lean_ctor_set(x_110, 1, x_100); +lean_ctor_set(x_110, 2, x_101); +lean_ctor_set(x_110, 3, x_102); +lean_ctor_set(x_110, 4, x_103); +lean_ctor_set(x_110, 5, x_104); +lean_ctor_set(x_110, 6, x_109); +x_111 = lean_st_ref_set(x_9, x_110, x_80); +lean_dec(x_9); +x_112 = lean_ctor_get(x_111, 1); +lean_inc(x_112); +if (lean_is_exclusive(x_111)) { + lean_ctor_release(x_111, 0); + lean_ctor_release(x_111, 1); + x_113 = x_111; +} else { + lean_dec_ref(x_111); + x_113 = lean_box(0); +} +if (lean_is_scalar(x_113)) { + x_114 = lean_alloc_ctor(1, 2, 0); +} else { + x_114 = x_113; + lean_ctor_set_tag(x_114, 1); +} +lean_ctor_set(x_114, 0, x_67); +lean_ctor_set(x_114, 1, x_112); +return x_114; +} +} +else +{ +uint8_t x_115; +lean_dec(x_67); +lean_dec(x_12); +lean_dec(x_9); +x_115 = !lean_is_exclusive(x_74); +if (x_115 == 0) +{ +return x_74; +} +else +{ +lean_object* x_116; lean_object* x_117; lean_object* x_118; +x_116 = lean_ctor_get(x_74, 0); +x_117 = lean_ctor_get(x_74, 1); +lean_inc(x_117); +lean_inc(x_116); +lean_dec(x_74); +x_118 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_118, 0, x_116); +lean_ctor_set(x_118, 1, x_117); +return x_118; +} +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_10 = lean_st_ref_get(x_8, x_9); +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_11, 6); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_ctor_get_uint8(x_12, sizeof(void*)*2); +lean_dec(x_12); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; +lean_dec(x_2); +x_14 = lean_ctor_get(x_10, 1); +lean_inc(x_14); +lean_dec(x_10); +x_15 = lean_apply_7(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_14); +if (lean_obj_tag(x_15) == 0) +{ +uint8_t x_16; +x_16 = !lean_is_exclusive(x_15); +if (x_16 == 0) +{ +return x_15; +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_15, 0); +x_18 = lean_ctor_get(x_15, 1); +lean_inc(x_18); +lean_inc(x_17); +lean_dec(x_15); +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set(x_19, 1, x_18); +return x_19; +} +} +else +{ +uint8_t x_20; +x_20 = !lean_is_exclusive(x_15); +if (x_20 == 0) +{ +return x_15; +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_15, 0); +x_22 = lean_ctor_get(x_15, 1); +lean_inc(x_22); +lean_inc(x_21); +lean_dec(x_15); +x_23 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_23, 0, x_21); +lean_ctor_set(x_23, 1, x_22); +return x_23; +} +} +} +else +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_10, 1); +lean_inc(x_24); +lean_dec(x_10); +x_25 = lean_box(0); +x_26 = l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__5___lambda__1(x_1, x_2, x_25, x_3, x_4, x_5, x_6, x_7, x_8, x_24); +return x_26; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_withSaveInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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) { +_start: +{ +lean_object* x_8; uint8_t x_9; +x_8 = l_Lean_Elab_CommandContextInfo_save___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_9 = !lean_is_exclusive(x_8); +if (x_9 == 0) +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_8, 0); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_12, 0, x_11); +lean_ctor_set(x_8, 0, x_12); +return x_8; +} +else +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_13 = lean_ctor_get(x_8, 0); +x_14 = lean_ctor_get(x_8, 1); +lean_inc(x_14); +lean_inc(x_13); +lean_dec(x_8); +x_15 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_15, 0, x_13); +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_14); +return x_17; +} +} +} +static lean_object* _init_l_Lean_Elab_withSaveInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__4___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_withSaveInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__4___lambda__1___boxed), 7, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_withSaveInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; lean_object* x_10; +x_9 = l_Lean_Elab_withSaveInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__4___closed__1; +x_10 = l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__5(x_1, x_9, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +return x_10; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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, 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) { +_start: +{ +lean_object* x_16; lean_object* x_17; +lean_inc(x_8); +x_16 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectLevelParamsInInductive(x_8); +x_17 = l_Lean_Elab_sortDeclLevelParams(x_1, x_2, x_16); +if (lean_obj_tag(x_17) == 0) +{ +uint8_t x_18; +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_5); +x_18 = !lean_is_exclusive(x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; +lean_ctor_set_tag(x_17, 3); +x_19 = l_Lean_MessageData_ofFormat(x_17); +x_20 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_19, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +return x_20; +} +else +{ +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(3, 1, 0); +lean_ctor_set(x_22, 0, x_21); +x_23 = l_Lean_MessageData_ofFormat(x_22); +x_24 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_23, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +return x_24; +} +} +else +{ +lean_object* x_25; lean_object* x_26; +x_25 = lean_ctor_get(x_17, 0); +lean_inc(x_25); +lean_dec(x_17); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_6); +lean_inc(x_25); +x_26 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_replaceIndFVarsWithConsts(x_3, x_4, x_25, x_5, x_6, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +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(6, 3, 1); +lean_ctor_set(x_29, 0, x_25); +lean_ctor_set(x_29, 1, x_6); +lean_ctor_set(x_29, 2, x_27); +lean_ctor_set_uint8(x_29, sizeof(void*)*3, x_7); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_29); +x_30 = l_Lean_Elab_Term_ensureNoUnassignedMVars(x_29, x_9, x_10, x_11, x_12, x_13, x_14, x_28); +if (lean_obj_tag(x_30) == 0) +{ +lean_object* x_31; lean_object* x_32; +x_31 = lean_ctor_get(x_30, 1); +lean_inc(x_31); +lean_dec(x_30); +lean_inc(x_14); +lean_inc(x_13); +x_32 = l_Lean_addDecl(x_29, x_13, x_14, x_31); +if (lean_obj_tag(x_32) == 0) +{ +lean_object* x_33; lean_object* x_34; +x_33 = lean_ctor_get(x_32, 1); +lean_inc(x_33); +lean_dec(x_32); +x_34 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions(x_3, x_9, x_10, x_11, x_12, x_13, x_14, x_33); +lean_dec(x_10); +lean_dec(x_9); +return x_34; +} +else +{ +uint8_t x_35; +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_35 = !lean_is_exclusive(x_32); +if (x_35 == 0) +{ +return x_32; +} +else +{ +lean_object* x_36; lean_object* x_37; lean_object* x_38; +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_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_29); +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_39 = !lean_is_exclusive(x_30); +if (x_39 == 0) +{ +return x_30; +} +else +{ +lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_40 = lean_ctor_get(x_30, 0); +x_41 = lean_ctor_get(x_30, 1); +lean_inc(x_41); +lean_inc(x_40); +lean_dec(x_30); +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_dec(x_25); +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_6); +x_43 = !lean_is_exclusive(x_26); +if (x_43 == 0) +{ +return x_26; +} +else +{ +lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_44 = lean_ctor_get(x_26, 0); +x_45 = lean_ctor_get(x_26, 1); +lean_inc(x_45); +lean_inc(x_44); +lean_dec(x_26); +x_46 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_46, 0, x_44); +lean_ctor_set(x_46, 1, x_45); +return x_46; +} +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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, uint8_t x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +_start: +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_array_get_size(x_9); +x_18 = lean_nat_add(x_17, x_1); +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_19 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateParams(x_9, x_2, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_19) == 0) +{ +if (lean_obj_tag(x_8) == 0) +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_19, 1); +lean_inc(x_21); +lean_dec(x_19); +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_20); +lean_inc(x_18); +lean_inc(x_5); +x_22 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses(x_5, x_18, x_20, x_10, x_11, x_12, x_13, x_14, x_15, x_21); +if (lean_obj_tag(x_22) == 0) +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_23 = lean_ctor_get(x_22, 1); +lean_inc(x_23); +lean_dec(x_22); +x_24 = lean_box(0); +x_25 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam(x_20, x_24, x_10, x_11, x_12, x_13, x_14, x_15, x_23); +x_26 = lean_ctor_get(x_25, 0); +lean_inc(x_26); +x_27 = lean_ctor_get(x_25, 1); +lean_inc(x_27); +lean_dec(x_25); +x_28 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__1(x_3, x_4, x_5, x_6, x_17, x_18, x_7, x_26, x_10, x_11, x_12, x_13, x_14, x_15, x_27); +lean_dec(x_5); +return x_28; +} +else +{ +uint8_t x_29; +lean_dec(x_20); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_29 = !lean_is_exclusive(x_22); +if (x_29 == 0) +{ +return x_22; +} +else +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_22, 0); +x_31 = lean_ctor_get(x_22, 1); +lean_inc(x_31); +lean_inc(x_30); +lean_dec(x_22); +x_32 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_31); +return x_32; +} +} +} +else +{ +lean_object* x_33; lean_object* x_34; uint8_t x_35; +x_33 = lean_ctor_get(x_19, 0); +lean_inc(x_33); +x_34 = lean_ctor_get(x_19, 1); +lean_inc(x_34); +lean_dec(x_19); +x_35 = !lean_is_exclusive(x_8); +if (x_35 == 0) +{ +lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_36 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam(x_33, x_8, x_10, x_11, x_12, x_13, x_14, x_15, x_34); +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_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_18); +x_39 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse(x_5, x_18, x_37, x_10, x_11, x_12, x_13, x_14, x_15, x_38); +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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__1(x_3, x_4, x_5, x_6, x_17, x_18, x_7, x_40, x_10, x_11, x_12, x_13, x_14, x_15, x_41); +lean_dec(x_5); +return x_42; +} +else +{ +uint8_t x_43; +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_43 = !lean_is_exclusive(x_39); +if (x_43 == 0) +{ +return x_39; +} +else +{ +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_object* x_50; lean_object* x_51; lean_object* x_52; +x_47 = lean_ctor_get(x_8, 0); +lean_inc(x_47); +lean_dec(x_8); +x_48 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_48, 0, x_47); +x_49 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam(x_33, x_48, x_10, x_11, x_12, x_13, x_14, x_15, x_34); +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_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_18); +x_52 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse(x_5, x_18, x_50, x_10, x_11, x_12, x_13, x_14, x_15, x_51); +if (lean_obj_tag(x_52) == 0) +{ +lean_object* x_53; lean_object* x_54; lean_object* x_55; +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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__1(x_3, x_4, x_5, x_6, x_17, x_18, x_7, x_53, x_10, x_11, x_12, x_13, x_14, x_15, x_54); +lean_dec(x_5); +return x_55; +} +else +{ +lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_56 = lean_ctor_get(x_52, 0); +lean_inc(x_56); +x_57 = lean_ctor_get(x_52, 1); +lean_inc(x_57); +if (lean_is_exclusive(x_52)) { + lean_ctor_release(x_52, 0); + lean_ctor_release(x_52, 1); + x_58 = x_52; +} else { + lean_dec_ref(x_52); + x_58 = lean_box(0); +} +if (lean_is_scalar(x_58)) { + x_59 = lean_alloc_ctor(1, 2, 0); +} else { + x_59 = x_58; +} +lean_ctor_set(x_59, 0, x_56); +lean_ctor_set(x_59, 1, x_57); +return x_59; +} +} +} +} +else +{ +uint8_t x_60; +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_60 = !lean_is_exclusive(x_19); +if (x_60 == 0) +{ +return x_19; +} +else +{ +lean_object* x_61; lean_object* x_62; lean_object* x_63; +x_61 = lean_ctor_get(x_19, 0); +x_62 = lean_ctor_get(x_19, 1); +lean_inc(x_62); +lean_inc(x_61); +lean_dec(x_19); +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; +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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, uint8_t x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +_start: +{ +lean_object* x_17; lean_object* x_18; +x_17 = lean_array_to_list(x_1); +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_17); +x_18 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse(x_17, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_18) == 0) +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; +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); +x_21 = l_Lean_Elab_Command_shouldInferResultUniverse(x_19, x_10, x_11, x_12, x_13, x_14, x_15, x_20); +if (lean_obj_tag(x_21) == 0) +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; 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_box(x_7); +lean_inc(x_17); +x_25 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__2___boxed), 16, 8); +lean_closure_set(x_25, 0, x_2); +lean_closure_set(x_25, 1, x_17); +lean_closure_set(x_25, 2, x_3); +lean_closure_set(x_25, 3, x_4); +lean_closure_set(x_25, 4, x_5); +lean_closure_set(x_25, 5, x_6); +lean_closure_set(x_25, 6, x_24); +lean_closure_set(x_25, 7, x_22); +x_26 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withUsed___rarg(x_8, x_17, x_25, x_10, x_11, x_12, x_13, x_14, x_15, x_23); +return x_26; +} +else +{ +uint8_t x_27; +lean_dec(x_17); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_27 = !lean_is_exclusive(x_21); +if (x_27 == 0) +{ +return x_21; +} +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; +} +} +} +else +{ +uint8_t x_31; +lean_dec(x_17); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_31 = !lean_is_exclusive(x_18); +if (x_31 == 0) +{ +return x_18; +} +else +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_18, 0); +x_33 = lean_ctor_get(x_18, 1); +lean_inc(x_33); +lean_inc(x_32); +lean_dec(x_18); +x_34 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_34, 0, x_32); +lean_ctor_set(x_34, 1, x_33); +return x_34; +} +} +} +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__4___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("numExplicitParams: ", 19, 19); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__4___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__4___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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, uint8_t x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18) { +_start: +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_19 = lean_array_get_size(x_1); +x_20 = lean_unsigned_to_nat(0u); +x_21 = lean_unsigned_to_nat(1u); +x_22 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__8___closed__1; +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_19); +lean_inc(x_5); +lean_inc(x_4); +x_23 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__1(x_1, x_2, x_3, x_4, x_5, x_19, x_19, x_20, x_19, x_21, x_22, x_12, x_13, x_14, x_15, x_16, x_17, x_18); +lean_dec(x_19); +if (lean_obj_tag(x_23) == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +x_26 = lean_array_get_size(x_4); +lean_dec(x_4); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_5); +lean_inc(x_24); +x_27 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams(x_26, x_24, x_5, x_14, x_15, x_16, x_17, x_25); +if (lean_obj_tag(x_27) == 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_27, 0); +lean_inc(x_28); +x_29 = lean_ctor_get(x_27, 1); +lean_inc(x_29); +lean_dec(x_27); +lean_inc(x_6); +x_30 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_6, x_12, x_13, x_14, x_15, x_16, x_17, x_29); +x_31 = lean_ctor_get(x_30, 0); +lean_inc(x_31); +x_32 = lean_unbox(x_31); +lean_dec(x_31); +if (x_32 == 0) +{ +lean_object* x_33; lean_object* x_34; lean_object* x_35; +lean_dec(x_6); +x_33 = lean_ctor_get(x_30, 1); +lean_inc(x_33); +lean_dec(x_30); +x_34 = lean_box(0); +x_35 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__3(x_24, x_28, x_7, x_8, x_1, x_5, x_9, x_10, x_34, x_12, x_13, x_14, x_15, x_16, x_17, x_33); +return x_35; +} +else +{ +uint8_t x_36; +x_36 = !lean_is_exclusive(x_30); +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; lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_37 = lean_ctor_get(x_30, 1); +x_38 = lean_ctor_get(x_30, 0); +lean_dec(x_38); +lean_inc(x_28); +x_39 = l___private_Init_Data_Repr_0__Nat_reprFast(x_28); +x_40 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_40, 0, x_39); +x_41 = l_Lean_MessageData_ofFormat(x_40); +x_42 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__4___closed__2; +lean_ctor_set_tag(x_30, 7); +lean_ctor_set(x_30, 1, x_41); +lean_ctor_set(x_30, 0, x_42); +x_43 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +x_44 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_44, 0, x_30); +lean_ctor_set(x_44, 1, x_43); +x_45 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_6, x_44, x_12, x_13, x_14, x_15, x_16, x_17, x_37); +x_46 = lean_ctor_get(x_45, 0); +lean_inc(x_46); +x_47 = lean_ctor_get(x_45, 1); +lean_inc(x_47); +lean_dec(x_45); +x_48 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__3(x_24, x_28, x_7, x_8, x_1, x_5, x_9, x_10, x_46, x_12, x_13, x_14, x_15, x_16, x_17, x_47); +lean_dec(x_46); +return x_48; +} +else +{ +lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; +x_49 = lean_ctor_get(x_30, 1); +lean_inc(x_49); +lean_dec(x_30); +lean_inc(x_28); +x_50 = l___private_Init_Data_Repr_0__Nat_reprFast(x_28); +x_51 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_51, 0, x_50); +x_52 = l_Lean_MessageData_ofFormat(x_51); +x_53 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__4___closed__2; +x_54 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_54, 0, x_53); +lean_ctor_set(x_54, 1, x_52); +x_55 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +x_56 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_56, 0, x_54); +lean_ctor_set(x_56, 1, x_55); +x_57 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_6, x_56, x_12, x_13, x_14, x_15, x_16, x_17, x_49); +x_58 = lean_ctor_get(x_57, 0); +lean_inc(x_58); +x_59 = lean_ctor_get(x_57, 1); +lean_inc(x_59); +lean_dec(x_57); +x_60 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__3(x_24, x_28, x_7, x_8, x_1, x_5, x_9, x_10, x_58, x_12, x_13, x_14, x_15, x_16, x_17, x_59); +lean_dec(x_58); +return x_60; +} +} +} +else +{ +uint8_t x_61; +lean_dec(x_24); +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_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_1); +x_61 = !lean_is_exclusive(x_27); +if (x_61 == 0) +{ +return x_27; +} +else +{ +lean_object* x_62; lean_object* x_63; lean_object* x_64; +x_62 = lean_ctor_get(x_27, 0); +x_63 = lean_ctor_get(x_27, 1); +lean_inc(x_63); +lean_inc(x_62); +lean_dec(x_27); +x_64 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_64, 0, x_62); +lean_ctor_set(x_64, 1, x_63); +return x_64; +} +} +} +else +{ +uint8_t x_65; +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_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_1); +x_65 = !lean_is_exclusive(x_23); +if (x_65 == 0) +{ +return x_23; +} +else +{ +lean_object* x_66; lean_object* x_67; lean_object* x_68; +x_66 = lean_ctor_get(x_23, 0); +x_67 = lean_ctor_get(x_23, 1); +lean_inc(x_67); +lean_inc(x_66); +lean_dec(x_23); +x_68 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_68, 0, x_66); +lean_ctor_set(x_68, 1, x_67); +return x_68; +} +} +} +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__5___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("indFVars: ", 10, 10); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__5___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__5___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, uint8_t x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { +_start: +{ +lean_object* x_18; lean_object* x_19; uint8_t x_20; +lean_inc(x_1); +x_18 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_1, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +x_20 = lean_unbox(x_19); +lean_dec(x_19); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_18, 1); +lean_inc(x_21); +lean_dec(x_18); +x_22 = lean_box(0); +x_23 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__4(x_2, x_3, x_4, x_9, x_10, x_1, x_5, x_6, x_7, x_8, x_22, x_11, x_12, x_13, x_14, x_15, x_16, x_21); +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; 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_18, 1); +x_26 = lean_ctor_get(x_18, 0); +lean_dec(x_26); +lean_inc(x_10); +x_27 = lean_array_to_list(x_10); +x_28 = lean_box(0); +x_29 = l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(x_27, x_28); +x_30 = l_Lean_MessageData_ofList(x_29); +x_31 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__5___closed__2; +lean_ctor_set_tag(x_18, 7); +lean_ctor_set(x_18, 1, x_30); +lean_ctor_set(x_18, 0, x_31); +x_32 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +x_33 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_33, 0, x_18); +lean_ctor_set(x_33, 1, x_32); +lean_inc(x_1); +x_34 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_1, x_33, x_11, x_12, x_13, x_14, x_15, x_16, x_25); +x_35 = lean_ctor_get(x_34, 0); +lean_inc(x_35); +x_36 = lean_ctor_get(x_34, 1); +lean_inc(x_36); +lean_dec(x_34); +x_37 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__4(x_2, x_3, x_4, x_9, x_10, x_1, x_5, x_6, x_7, x_8, x_35, x_11, x_12, x_13, x_14, x_15, x_16, x_36); +lean_dec(x_35); +return x_37; +} +else +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_38 = lean_ctor_get(x_18, 1); +lean_inc(x_38); +lean_dec(x_18); +lean_inc(x_10); +x_39 = lean_array_to_list(x_10); +x_40 = lean_box(0); +x_41 = l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(x_39, x_40); +x_42 = l_Lean_MessageData_ofList(x_41); +x_43 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__5___closed__2; +x_44 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_44, 0, x_43); +lean_ctor_set(x_44, 1, x_42); +x_45 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +x_46 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_46, 0, x_44); +lean_ctor_set(x_46, 1, x_45); +lean_inc(x_1); +x_47 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_1, x_46, x_11, x_12, x_13, x_14, x_15, x_16, x_38); +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_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__4(x_2, x_3, x_4, x_9, x_10, x_1, x_5, x_6, x_7, x_8, x_48, x_11, x_12, x_13, x_14, x_15, x_16, x_49); +lean_dec(x_48); +return x_50; +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__6(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; +x_11 = lean_box(0); +x_12 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__3(x_1, x_2, x_3, x_11, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_12) == 0) +{ +uint8_t x_13; +x_13 = !lean_is_exclusive(x_12); +if (x_13 == 0) +{ +lean_object* x_14; +x_14 = lean_ctor_get(x_12, 0); +lean_dec(x_14); +lean_ctor_set(x_12, 0, x_11); +return x_12; +} +else +{ +lean_object* x_15; lean_object* x_16; +x_15 = lean_ctor_get(x_12, 1); +lean_inc(x_15); +lean_dec(x_12); +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_11); +lean_ctor_set(x_16, 1, x_15); +return x_16; +} +} +else +{ +uint8_t x_17; +x_17 = !lean_is_exclusive(x_12); +if (x_17 == 0) +{ +return x_12; +} +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; +} +} +} +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__7___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_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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, uint8_t x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +_start: +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_box(x_7); +lean_inc(x_3); +lean_inc(x_2); +x_18 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__5___boxed), 17, 8); +lean_closure_set(x_18, 0, x_1); +lean_closure_set(x_18, 1, x_2); +lean_closure_set(x_18, 2, x_3); +lean_closure_set(x_18, 3, x_4); +lean_closure_set(x_18, 4, x_5); +lean_closure_set(x_18, 5, x_6); +lean_closure_set(x_18, 6, x_17); +lean_closure_set(x_18, 7, x_8); +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_19 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withInductiveLocalDecls___rarg(x_3, x_18, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_19) == 0) +{ +lean_object* 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; +x_20 = lean_ctor_get(x_19, 1); +lean_inc(x_20); +lean_dec(x_19); +x_21 = lean_array_size(x_2); +x_22 = lean_box_usize(x_21); +x_23 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__7___boxed__const__1; +x_24 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__6___boxed), 10, 3); +lean_closure_set(x_24, 0, x_2); +lean_closure_set(x_24, 1, x_22); +lean_closure_set(x_24, 2, x_23); +x_25 = lean_alloc_closure((void*)(l_Lean_Elab_withSaveInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__4___lambda__1___boxed), 7, 0); +x_26 = l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__5(x_24, x_25, x_10, x_11, x_12, x_13, x_14, x_15, x_20); +return x_26; +} +else +{ +uint8_t x_27; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_2); +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; +} +} +} +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__8___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("level names: ", 13, 13); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__8___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__8___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__8(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_1); +x_12 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeader(x_1, 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; uint8_t x_15; uint8_t x_16; lean_object* x_17; +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_12, 1); +lean_inc(x_14); +lean_dec(x_12); +x_15 = 1; +x_16 = 0; +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_17 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_15, x_16, x_5, x_6, x_7, x_8, x_9, x_10, x_14); +if (lean_obj_tag(x_17) == 0) +{ +lean_object* x_18; lean_object* x_19; +x_18 = lean_ctor_get(x_17, 1); +lean_inc(x_18); +lean_dec(x_17); +lean_inc(x_9); +lean_inc(x_5); +x_19 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_ElabHeaderResult_checkLevelNames(x_13, 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; uint8_t x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_20 = lean_ctor_get(x_19, 1); +lean_inc(x_20); +lean_dec(x_19); +x_21 = lean_array_get_size(x_13); +x_22 = lean_unsigned_to_nat(0u); +x_23 = lean_nat_dec_lt(x_22, x_21); +x_24 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__3; +x_25 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_24, x_5, x_6, x_7, x_8, x_9, x_10, x_20); +if (x_23 == 0) +{ +lean_object* x_61; lean_object* x_62; +x_61 = l_Lean_Elab_Command_instInhabitedElabHeaderResult; +x_62 = l_outOfBounds___rarg(x_61); +x_26 = x_62; +goto block_60; +} +else +{ +lean_object* x_63; +x_63 = lean_array_fget(x_13, x_22); +x_26 = x_63; +goto block_60; +} +block_60: +{ +lean_object* x_27; uint8_t x_28; +x_27 = lean_ctor_get(x_25, 0); +lean_inc(x_27); +x_28 = lean_unbox(x_27); +lean_dec(x_27); +if (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_25, 1); +lean_inc(x_29); +lean_dec(x_25); +x_30 = lean_ctor_get(x_26, 3); +lean_inc(x_30); +lean_dec(x_26); +x_31 = lean_box(0); +x_32 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__7(x_24, x_1, x_13, x_21, x_2, x_30, x_3, x_4, x_31, x_5, x_6, x_7, x_8, x_9, x_10, x_29); +return x_32; +} +else +{ +uint8_t x_33; +x_33 = !lean_is_exclusive(x_25); +if (x_33 == 0) +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_34 = lean_ctor_get(x_25, 1); +x_35 = lean_ctor_get(x_25, 0); +lean_dec(x_35); +x_36 = lean_ctor_get(x_26, 3); +lean_inc(x_36); +lean_dec(x_26); +x_37 = lean_box(0); +lean_inc(x_36); +x_38 = l_List_mapTR_loop___at_Lean_compileDecl___spec__1(x_36, x_37); +x_39 = l_Lean_MessageData_ofList(x_38); +x_40 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__8___closed__2; +lean_ctor_set_tag(x_25, 7); +lean_ctor_set(x_25, 1, x_39); +lean_ctor_set(x_25, 0, x_40); +x_41 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +x_42 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_42, 0, x_25); +lean_ctor_set(x_42, 1, x_41); +x_43 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_24, x_42, x_5, x_6, x_7, x_8, x_9, x_10, x_34); +x_44 = lean_ctor_get(x_43, 0); +lean_inc(x_44); +x_45 = lean_ctor_get(x_43, 1); +lean_inc(x_45); +lean_dec(x_43); +x_46 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__7(x_24, x_1, x_13, x_21, x_2, x_36, x_3, x_4, x_44, x_5, x_6, x_7, x_8, x_9, x_10, x_45); +lean_dec(x_44); +return x_46; +} +else +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_47 = lean_ctor_get(x_25, 1); +lean_inc(x_47); +lean_dec(x_25); +x_48 = lean_ctor_get(x_26, 3); +lean_inc(x_48); +lean_dec(x_26); +x_49 = lean_box(0); +lean_inc(x_48); +x_50 = l_List_mapTR_loop___at_Lean_compileDecl___spec__1(x_48, x_49); +x_51 = l_Lean_MessageData_ofList(x_50); +x_52 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__8___closed__2; +x_53 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_53, 0, x_52); +lean_ctor_set(x_53, 1, x_51); +x_54 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +x_55 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_55, 0, x_53); +lean_ctor_set(x_55, 1, x_54); +x_56 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_24, x_55, x_5, x_6, x_7, x_8, x_9, x_10, x_47); +x_57 = lean_ctor_get(x_56, 0); +lean_inc(x_57); +x_58 = lean_ctor_get(x_56, 1); +lean_inc(x_58); +lean_dec(x_56); +x_59 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__7(x_24, x_1, x_13, x_21, x_2, x_48, x_3, x_4, x_57, x_5, x_6, x_7, x_8, x_9, x_10, x_58); +lean_dec(x_57); +return x_59; +} +} +} +} +else +{ +uint8_t x_64; +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_2); +lean_dec(x_1); +x_64 = !lean_is_exclusive(x_19); +if (x_64 == 0) +{ +return x_19; +} +else +{ +lean_object* x_65; lean_object* x_66; lean_object* x_67; +x_65 = lean_ctor_get(x_19, 0); +x_66 = lean_ctor_get(x_19, 1); +lean_inc(x_66); +lean_inc(x_65); +lean_dec(x_19); +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_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_2); +lean_dec(x_1); +x_68 = !lean_is_exclusive(x_17); +if (x_68 == 0) +{ +return x_17; +} +else +{ +lean_object* x_69; lean_object* x_70; lean_object* x_71; +x_69 = lean_ctor_get(x_17, 0); +x_70 = lean_ctor_get(x_17, 1); +lean_inc(x_70); +lean_inc(x_69); +lean_dec(x_17); +x_71 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_71, 0, x_69); +lean_ctor_set(x_71, 1, x_70); +return x_71; +} +} +} +else +{ +uint8_t x_72; +lean_dec(x_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_72 = !lean_is_exclusive(x_12); +if (x_72 == 0) +{ +return x_12; +} +else +{ +lean_object* x_73; lean_object* x_74; lean_object* x_75; +x_73 = lean_ctor_get(x_12, 0); +x_74 = lean_ctor_get(x_12, 1); +lean_inc(x_74); +lean_inc(x_73); +lean_dec(x_12); +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_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +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); +lean_inc(x_8); +lean_inc(x_4); +x_14 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_InductiveView_checkLevelNames(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +if (lean_obj_tag(x_14) == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; +x_15 = lean_ctor_get(x_14, 1); +lean_inc(x_15); +lean_dec(x_14); +x_16 = lean_ctor_get(x_2, 5); +lean_inc(x_16); +x_17 = lean_ctor_get(x_2, 2); +lean_inc(x_17); +x_18 = lean_ctor_get_uint8(x_17, sizeof(void*)*3 + 3); +lean_dec(x_17); +x_19 = lean_ctor_get(x_2, 0); +lean_inc(x_19); +lean_dec(x_2); +x_20 = lean_box(x_18); +x_21 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__8___boxed), 11, 4); +lean_closure_set(x_21, 0, x_1); +lean_closure_set(x_21, 1, x_12); +lean_closure_set(x_21, 2, x_20); +lean_closure_set(x_21, 3, x_3); +x_22 = !lean_is_exclusive(x_8); +if (x_22 == 0) +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_8, 5); +x_24 = l_Lean_replaceRef(x_19, x_23); +lean_dec(x_23); +lean_dec(x_19); +lean_ctor_set(x_8, 5, x_24); +x_25 = l_Lean_Elab_Term_withLevelNames___rarg(x_16, x_21, x_4, x_5, x_6, x_7, x_8, x_9, x_15); +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_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; lean_object* x_38; uint8_t x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_26 = lean_ctor_get(x_8, 0); +x_27 = lean_ctor_get(x_8, 1); +x_28 = lean_ctor_get(x_8, 2); +x_29 = lean_ctor_get(x_8, 3); +x_30 = lean_ctor_get(x_8, 4); +x_31 = lean_ctor_get(x_8, 5); +x_32 = lean_ctor_get(x_8, 6); +x_33 = lean_ctor_get(x_8, 7); +x_34 = lean_ctor_get(x_8, 8); +x_35 = lean_ctor_get(x_8, 9); +x_36 = lean_ctor_get(x_8, 10); +x_37 = lean_ctor_get_uint8(x_8, sizeof(void*)*12); +x_38 = lean_ctor_get(x_8, 11); +x_39 = lean_ctor_get_uint8(x_8, sizeof(void*)*12 + 1); +lean_inc(x_38); +lean_inc(x_36); +lean_inc(x_35); +lean_inc(x_34); +lean_inc(x_33); +lean_inc(x_32); +lean_inc(x_31); +lean_inc(x_30); +lean_inc(x_29); +lean_inc(x_28); +lean_inc(x_27); +lean_inc(x_26); +lean_dec(x_8); +x_40 = l_Lean_replaceRef(x_19, x_31); +lean_dec(x_31); +lean_dec(x_19); +x_41 = lean_alloc_ctor(0, 12, 2); +lean_ctor_set(x_41, 0, x_26); +lean_ctor_set(x_41, 1, x_27); +lean_ctor_set(x_41, 2, x_28); +lean_ctor_set(x_41, 3, x_29); +lean_ctor_set(x_41, 4, x_30); +lean_ctor_set(x_41, 5, x_40); +lean_ctor_set(x_41, 6, x_32); +lean_ctor_set(x_41, 7, x_33); +lean_ctor_set(x_41, 8, x_34); +lean_ctor_set(x_41, 9, x_35); +lean_ctor_set(x_41, 10, x_36); +lean_ctor_set(x_41, 11, x_38); +lean_ctor_set_uint8(x_41, sizeof(void*)*12, x_37); +lean_ctor_set_uint8(x_41, sizeof(void*)*12 + 1, x_39); +x_42 = l_Lean_Elab_Term_withLevelNames___rarg(x_16, x_21, x_4, x_5, x_6, x_7, x_41, x_9, x_15); +return x_42; +} +} +else +{ +uint8_t x_43; +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_43 = !lean_is_exclusive(x_14); +if (x_43 == 0) +{ +return x_14; +} +else +{ +lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_44 = lean_ctor_get(x_14, 0); +x_45 = lean_ctor_get(x_14, 1); +lean_inc(x_45); +lean_inc(x_44); +lean_dec(x_14); +x_46 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_46, 0, x_44); +lean_ctor_set(x_46, 1, x_45); +return x_46; +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; uint8_t x_12; +x_10 = lean_array_get_size(x_2); +x_11 = lean_unsigned_to_nat(0u); +x_12 = lean_nat_dec_lt(x_11, x_10); +lean_dec(x_10); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_13 = l_Lean_Elab_Command_instInhabitedInductiveView; +x_14 = l_outOfBounds___rarg(x_13); +x_15 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__9), 10, 3); +lean_closure_set(x_15, 0, x_2); +lean_closure_set(x_15, 1, x_14); +lean_closure_set(x_15, 2, x_1); +x_16 = l_Lean_Elab_Term_withoutSavingRecAppSyntax___rarg(x_15, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_16; +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_array_fget(x_2, x_11); +x_18 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__9), 10, 3); +lean_closure_set(x_18, 0, x_2); +lean_closure_set(x_18, 1, x_17); +lean_closure_set(x_18, 2, x_1); +x_19 = l_Lean_Elab_Term_withoutSavingRecAppSyntax___rarg(x_18, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_19; +} +} +} +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__1___boxed(lean_object** _args) { +lean_object* x_1 = _args[0]; +lean_object* x_2 = _args[1]; +lean_object* x_3 = _args[2]; +lean_object* x_4 = _args[3]; +lean_object* x_5 = _args[4]; +lean_object* x_6 = _args[5]; +lean_object* x_7 = _args[6]; +lean_object* x_8 = _args[7]; +lean_object* x_9 = _args[8]; +lean_object* x_10 = _args[9]; +lean_object* x_11 = _args[10]; +lean_object* x_12 = _args[11]; +lean_object* x_13 = _args[12]; +lean_object* x_14 = _args[13]; +lean_object* x_15 = _args[14]; +lean_object* x_16 = _args[15]; +lean_object* x_17 = _args[16]; +lean_object* x_18 = _args[17]; +_start: +{ +lean_object* x_19; +x_19 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_19; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +size_t x_14; size_t x_15; lean_object* x_16; +x_14 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_15 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_16 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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_3); +return x_16; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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; +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_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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_1); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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) { +_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_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__8(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +return x_15; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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_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_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__9(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +return x_15; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +size_t x_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_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__10(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +return x_15; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, 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_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__13(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +return x_15; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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_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_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__14(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +return x_15; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__15___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_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_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__15(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +return x_15; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__5___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_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_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__5___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_3); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_withSaveInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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) { +_start: +{ +lean_object* x_8; +x_8 = l_Lean_Elab_withSaveInfoContext___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__4___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_8; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, 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_7); +lean_dec(x_7); +x_17 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_16, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +lean_dec(x_4); +lean_dec(x_3); +return x_17; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +_start: +{ +uint8_t x_17; lean_object* x_18; +x_17 = lean_unbox(x_7); +lean_dec(x_7); +x_18 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_17, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +lean_dec(x_6); +lean_dec(x_1); +return x_18; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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_7); +lean_dec(x_7); +x_18 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_17, 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_8); +return x_18; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__4___boxed(lean_object** _args) { +lean_object* x_1 = _args[0]; +lean_object* x_2 = _args[1]; +lean_object* x_3 = _args[2]; +lean_object* x_4 = _args[3]; +lean_object* x_5 = _args[4]; +lean_object* x_6 = _args[5]; +lean_object* x_7 = _args[6]; +lean_object* x_8 = _args[7]; +lean_object* x_9 = _args[8]; +lean_object* x_10 = _args[9]; +lean_object* x_11 = _args[10]; +lean_object* x_12 = _args[11]; +lean_object* x_13 = _args[12]; +lean_object* x_14 = _args[13]; +lean_object* x_15 = _args[14]; +lean_object* x_16 = _args[15]; +lean_object* x_17 = _args[16]; +lean_object* x_18 = _args[17]; +_start: +{ +uint8_t x_19; lean_object* x_20; +x_19 = lean_unbox(x_9); +lean_dec(x_9); +x_20 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_19, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_3); +lean_dec(x_2); +return x_20; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___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: +{ +uint8_t x_18; lean_object* x_19; +x_18 = lean_unbox(x_7); +lean_dec(x_7); +x_19 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_18, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +lean_dec(x_8); +lean_dec(x_4); +lean_dec(x_3); +return x_19; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +size_t x_11; size_t x_12; lean_object* x_13; +x_11 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_12 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_13 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__6(x_1, x_11, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_1); +return x_13; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +_start: +{ +uint8_t x_17; lean_object* x_18; +x_17 = lean_unbox(x_7); +lean_dec(x_7); +x_18 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__7(x_1, x_2, x_3, x_4, x_5, x_6, x_17, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +lean_dec(x_9); +return x_18; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +uint8_t x_12; lean_object* x_13; +x_12 = lean_unbox(x_3); +lean_dec(x_3); +x_13 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__8(x_1, x_2, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_13; +} +} +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___spec__1(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; lean_object* x_7; uint8_t x_8; +x_6 = lean_array_uget(x_2, x_3); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +x_8 = lean_name_eq(x_7, x_1); +lean_dec(x_7); +if (x_8 == 0) +{ +size_t x_9; size_t x_10; +x_9 = 1; +x_10 = lean_usize_add(x_3, x_9); +x_3 = x_10; +goto _start; +} +else +{ +uint8_t x_12; +x_12 = 1; +return x_12; +} +} +else +{ +uint8_t x_13; +x_13 = 0; +return x_13; +} +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___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) { +_start: +{ +uint8_t x_9; +x_9 = lean_usize_dec_lt(x_4, x_3); +if (x_9 == 0) +{ +lean_object* x_10; +x_10 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_10, 0, x_5); +lean_ctor_set(x_10, 1, x_8); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_11 = lean_array_uget(x_2, x_4); +x_12 = lean_ctor_get(x_11, 9); +lean_inc(x_12); +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); +if (x_15 == 0) +{ +size_t x_16; size_t x_17; +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +x_16 = 1; +x_17 = lean_usize_add(x_4, x_16); +x_4 = x_17; +goto _start; +} +else +{ +size_t x_19; size_t x_20; uint8_t x_21; +x_19 = 0; +x_20 = lean_usize_of_nat(x_13); +lean_dec(x_13); +x_21 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___spec__1(x_1, x_12, x_19, x_20); +lean_dec(x_12); +if (x_21 == 0) +{ +size_t x_22; size_t x_23; +lean_dec(x_11); +x_22 = 1; +x_23 = lean_usize_add(x_4, x_22); +x_4 = x_23; +goto _start; +} +else +{ +lean_object* x_25; lean_object* x_26; size_t x_27; size_t x_28; +x_25 = lean_ctor_get(x_11, 4); +lean_inc(x_25); +lean_dec(x_11); +x_26 = lean_array_push(x_5, x_25); +x_27 = 1; +x_28 = lean_usize_add(x_4, x_27); +x_4 = x_28; +x_5 = x_26; +goto _start; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___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) { +_start: +{ +uint8_t x_9; +x_9 = lean_usize_dec_lt(x_4, x_3); +if (x_9 == 0) +{ +lean_object* x_10; +lean_dec(x_7); +lean_dec(x_6); +x_10 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_10, 0, x_5); +lean_ctor_set(x_10, 1, x_8); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_11 = lean_array_uget(x_2, x_4); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +x_13 = l_Lean_NameSet_contains(x_5, x_12); +if (x_13 == 0) +{ +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; +x_14 = lean_box(0); +lean_inc(x_12); +x_15 = l_Lean_RBNode_insert___at_Lean_NameSet_insert___spec__1(x_5, x_12, x_14); +x_16 = lean_array_size(x_1); +x_17 = 0; +x_18 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__8___closed__1; +x_19 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___spec__2(x_12, x_1, x_16, x_17, x_18, x_6, x_7, x_8); +lean_dec(x_12); +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_19, 1); +lean_inc(x_21); +lean_dec(x_19); +lean_inc(x_7); +lean_inc(x_6); +x_22 = l_Lean_Elab_DerivingClassView_applyHandlers(x_11, x_20, x_6, x_7, x_21); +if (lean_obj_tag(x_22) == 0) +{ +lean_object* x_23; size_t x_24; size_t x_25; +x_23 = lean_ctor_get(x_22, 1); +lean_inc(x_23); +lean_dec(x_22); +x_24 = 1; +x_25 = lean_usize_add(x_4, x_24); +x_4 = x_25; +x_5 = x_15; +x_8 = x_23; +goto _start; +} +else +{ +uint8_t x_27; +lean_dec(x_15); +lean_dec(x_7); +lean_dec(x_6); +x_27 = !lean_is_exclusive(x_22); +if (x_27 == 0) +{ +return x_22; +} +else +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_22, 0); +x_29 = lean_ctor_get(x_22, 1); +lean_inc(x_29); +lean_inc(x_28); +lean_dec(x_22); +x_30 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +return x_30; +} +} +} +else +{ +size_t x_31; size_t x_32; +lean_dec(x_12); +lean_dec(x_11); +x_31 = 1; +x_32 = lean_usize_add(x_4, x_31); +x_4 = x_32; +goto _start; +} +} +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___spec__4(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) { +_start: +{ +uint8_t x_9; +x_9 = lean_usize_dec_lt(x_4, x_3); +if (x_9 == 0) +{ +lean_object* x_10; +lean_dec(x_7); +lean_dec(x_6); +x_10 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_10, 0, x_5); +lean_ctor_set(x_10, 1, x_8); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; size_t x_13; size_t x_14; lean_object* x_15; +x_11 = lean_array_uget(x_2, x_4); +x_12 = lean_ctor_get(x_11, 9); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_array_size(x_12); +x_14 = 0; +lean_inc(x_7); +lean_inc(x_6); +x_15 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___spec__3(x_1, x_12, x_13, x_14, x_5, x_6, x_7, x_8); +lean_dec(x_12); +if (lean_obj_tag(x_15) == 0) +{ +lean_object* x_16; lean_object* x_17; size_t x_18; size_t 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 = 1; +x_19 = lean_usize_add(x_4, x_18); +x_4 = x_19; +x_5 = x_16; +x_8 = x_17; +goto _start; +} +else +{ +uint8_t x_21; +lean_dec(x_7); +lean_dec(x_6); +x_21 = !lean_is_exclusive(x_15); +if (x_21 == 0) +{ +return x_15; +} +else +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_15, 0); +x_23 = lean_ctor_get(x_15, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_15); +x_24 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); +return x_24; +} +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers(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; lean_object* x_8; +x_5 = lean_array_size(x_1); +x_6 = 0; +x_7 = l_Lean_NameSet_empty; +x_8 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___spec__4(x_1, x_1, x_5, x_6, x_7, x_2, x_3, x_4); +if (lean_obj_tag(x_8) == 0) +{ +uint8_t x_9; +x_9 = !lean_is_exclusive(x_8); +if (x_9 == 0) +{ +lean_object* x_10; lean_object* x_11; +x_10 = lean_ctor_get(x_8, 0); +lean_dec(x_10); +x_11 = lean_box(0); +lean_ctor_set(x_8, 0, x_11); +return x_8; +} +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_8, 1); +lean_inc(x_12); +lean_dec(x_8); +x_13 = lean_box(0); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_13); +lean_ctor_set(x_14, 1, x_12); +return x_14; +} +} +else +{ +uint8_t x_15; +x_15 = !lean_is_exclusive(x_8); +if (x_15 == 0) +{ +return x_8; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_8, 0); +x_17 = lean_ctor_get(x_8, 1); +lean_inc(x_17); +lean_inc(x_16); +lean_dec(x_8); +x_18 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_18, 0, x_16); +lean_ctor_set(x_18, 1, x_17); +return x_18; +} +} +} +} +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___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; +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_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___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_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___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) { +_start: +{ +size_t x_9; size_t x_10; lean_object* x_11; +x_9 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_10 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_11 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___spec__2(x_1, x_2, x_9, x_10, x_5, x_6, x_7, x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_2); +lean_dec(x_1); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___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: +{ +size_t x_9; size_t x_10; lean_object* x_11; +x_9 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_10 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_11 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___spec__3(x_1, x_2, x_9, x_10, x_5, x_6, x_7, x_8); +lean_dec(x_2); +lean_dec(x_1); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +size_t x_9; size_t x_10; lean_object* x_11; +x_9 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_10 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_11 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___spec__4(x_1, x_2, x_9, x_10, x_5, x_6, x_7, x_8); +lean_dec(x_2); +lean_dec(x_1); +return x_11; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___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_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers(x_1, x_2, x_3, x_4); +lean_dec(x_1); +return x_5; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("declaration", 11, 11); +return x_1; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; +x_2 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__1; +x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__7; +x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__1; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("definition", 10, 10); +return x_1; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; +x_2 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__1; +x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__7; +x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__3; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("def", 3, 3); +return x_1; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("declId", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; +x_2 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__1; +x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__7; +x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__6; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__8() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("_root_", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___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_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__8; +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_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__10() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("optDeclSig", 10, 10); +return x_1; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__11() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; +x_2 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__1; +x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__7; +x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__10; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__12() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("typeSpec", 8, 8); +return x_1; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__13() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; +x_2 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__1; +x_3 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__1___closed__1; +x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__12; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__14() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(":", 1, 1); +return x_1; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__15() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("declValEqns", 11, 11); +return x_1; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__16() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; +x_2 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__1; +x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__7; +x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__15; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__17() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("matchAltsWhereDecls", 19, 19); +return x_1; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__18() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; +x_2 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__1; +x_3 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__1___closed__1; +x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__17; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__19() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Termination", 11, 11); +return x_1; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__20() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("suffix", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__21() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; +x_2 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__1; +x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__19; +x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__20; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___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; uint8_t x_11; +x_10 = l_Lean_Elab_Command_getRef(x_7, x_8, x_9); +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; uint8_t x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_12 = lean_ctor_get(x_10, 0); +x_13 = lean_ctor_get(x_10, 1); +x_14 = 0; +x_15 = l_Lean_SourceInfo_fromRef(x_12, x_14); +lean_dec(x_12); +x_16 = l_Lean_Elab_Command_getCurrMacroScope(x_7, x_8, x_13); +x_17 = !lean_is_exclusive(x_16); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_18 = lean_ctor_get(x_16, 1); +x_19 = lean_ctor_get(x_16, 0); +lean_dec(x_19); +x_20 = l_Lean_Elab_Command_getMainModule___rarg(x_8, x_18); +x_21 = !lean_is_exclusive(x_20); +if (x_21 == 0) +{ +lean_object* x_22; uint8_t x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_22 = lean_ctor_get(x_20, 0); +lean_dec(x_22); +x_23 = 1; +x_24 = l_Lean_SourceInfo_fromRef(x_1, x_23); +x_25 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__5; +lean_ctor_set_tag(x_16, 2); +lean_ctor_set(x_16, 1, x_25); +lean_ctor_set(x_16, 0, x_24); +x_26 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__9; +x_27 = l_Lean_Name_append(x_26, x_2); +x_28 = l_Lean_Name_append(x_27, x_3); +x_29 = lean_mk_syntax_ident(x_28); +x_30 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2; +x_31 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; +lean_inc(x_15); +x_32 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_32, 0, x_15); +lean_ctor_set(x_32, 1, x_30); +lean_ctor_set(x_32, 2, x_31); +x_33 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__7; +lean_inc(x_32); +lean_inc(x_15); +x_34 = l_Lean_Syntax_node2(x_15, x_33, x_29, x_32); +x_35 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__14; +lean_inc(x_15); +lean_ctor_set_tag(x_10, 2); +lean_ctor_set(x_10, 1, x_35); +lean_ctor_set(x_10, 0, x_15); +x_36 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__13; +lean_inc(x_15); +x_37 = l_Lean_Syntax_node2(x_15, x_36, x_10, x_4); +lean_inc(x_15); +x_38 = l_Lean_Syntax_node1(x_15, x_30, x_37); +x_39 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__11; +lean_inc(x_32); +lean_inc(x_15); +x_40 = l_Lean_Syntax_node2(x_15, x_39, x_32, x_38); +x_41 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__21; +lean_inc_n(x_32, 2); +lean_inc(x_15); +x_42 = l_Lean_Syntax_node2(x_15, x_41, x_32, x_32); +x_43 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__18; +lean_inc(x_32); +lean_inc(x_15); +x_44 = l_Lean_Syntax_node3(x_15, x_43, x_5, x_42, x_32); +x_45 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__16; +lean_inc(x_15); +x_46 = l_Lean_Syntax_node1(x_15, x_45, x_44); +x_47 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__4; +lean_inc(x_15); +x_48 = l_Lean_Syntax_node5(x_15, x_47, x_16, x_34, x_40, x_46, x_32); +x_49 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__2; +x_50 = l_Lean_Syntax_node2(x_15, x_49, x_6, x_48); +lean_ctor_set(x_20, 0, x_50); +return x_20; +} +else +{ +lean_object* x_51; uint8_t x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; +x_51 = lean_ctor_get(x_20, 1); +lean_inc(x_51); +lean_dec(x_20); +x_52 = 1; +x_53 = l_Lean_SourceInfo_fromRef(x_1, x_52); +x_54 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__5; +lean_ctor_set_tag(x_16, 2); +lean_ctor_set(x_16, 1, x_54); +lean_ctor_set(x_16, 0, x_53); +x_55 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__9; +x_56 = l_Lean_Name_append(x_55, x_2); +x_57 = l_Lean_Name_append(x_56, x_3); +x_58 = lean_mk_syntax_ident(x_57); +x_59 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2; +x_60 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; +lean_inc(x_15); +x_61 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_61, 0, x_15); +lean_ctor_set(x_61, 1, x_59); +lean_ctor_set(x_61, 2, x_60); +x_62 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__7; +lean_inc(x_61); +lean_inc(x_15); +x_63 = l_Lean_Syntax_node2(x_15, x_62, x_58, x_61); +x_64 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__14; +lean_inc(x_15); +lean_ctor_set_tag(x_10, 2); +lean_ctor_set(x_10, 1, x_64); +lean_ctor_set(x_10, 0, x_15); +x_65 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__13; +lean_inc(x_15); +x_66 = l_Lean_Syntax_node2(x_15, x_65, x_10, x_4); +lean_inc(x_15); +x_67 = l_Lean_Syntax_node1(x_15, x_59, x_66); +x_68 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__11; +lean_inc(x_61); +lean_inc(x_15); +x_69 = l_Lean_Syntax_node2(x_15, x_68, x_61, x_67); +x_70 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__21; +lean_inc_n(x_61, 2); +lean_inc(x_15); +x_71 = l_Lean_Syntax_node2(x_15, x_70, x_61, x_61); +x_72 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__18; +lean_inc(x_61); +lean_inc(x_15); +x_73 = l_Lean_Syntax_node3(x_15, x_72, x_5, x_71, x_61); +x_74 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__16; +lean_inc(x_15); +x_75 = l_Lean_Syntax_node1(x_15, x_74, x_73); +x_76 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__4; +lean_inc(x_15); +x_77 = l_Lean_Syntax_node5(x_15, x_76, x_16, x_63, x_69, x_75, x_61); +x_78 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__2; +x_79 = l_Lean_Syntax_node2(x_15, x_78, x_6, x_77); +x_80 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_80, 0, x_79); +lean_ctor_set(x_80, 1, x_51); +return x_80; +} +} +else +{ +lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; uint8_t x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; +x_81 = lean_ctor_get(x_16, 1); +lean_inc(x_81); +lean_dec(x_16); +x_82 = l_Lean_Elab_Command_getMainModule___rarg(x_8, x_81); +x_83 = lean_ctor_get(x_82, 1); +lean_inc(x_83); +if (lean_is_exclusive(x_82)) { + lean_ctor_release(x_82, 0); + lean_ctor_release(x_82, 1); + x_84 = x_82; +} else { + lean_dec_ref(x_82); + x_84 = lean_box(0); +} +x_85 = 1; +x_86 = l_Lean_SourceInfo_fromRef(x_1, x_85); +x_87 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__5; +x_88 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_88, 0, x_86); +lean_ctor_set(x_88, 1, x_87); +x_89 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__9; +x_90 = l_Lean_Name_append(x_89, x_2); +x_91 = l_Lean_Name_append(x_90, x_3); +x_92 = lean_mk_syntax_ident(x_91); +x_93 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2; +x_94 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; +lean_inc(x_15); +x_95 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_95, 0, x_15); +lean_ctor_set(x_95, 1, x_93); +lean_ctor_set(x_95, 2, x_94); +x_96 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__7; +lean_inc(x_95); +lean_inc(x_15); +x_97 = l_Lean_Syntax_node2(x_15, x_96, x_92, x_95); +x_98 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__14; +lean_inc(x_15); +lean_ctor_set_tag(x_10, 2); +lean_ctor_set(x_10, 1, x_98); +lean_ctor_set(x_10, 0, x_15); +x_99 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__13; +lean_inc(x_15); +x_100 = l_Lean_Syntax_node2(x_15, x_99, x_10, x_4); +lean_inc(x_15); +x_101 = l_Lean_Syntax_node1(x_15, x_93, x_100); +x_102 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__11; +lean_inc(x_95); +lean_inc(x_15); +x_103 = l_Lean_Syntax_node2(x_15, x_102, x_95, x_101); +x_104 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__21; +lean_inc_n(x_95, 2); +lean_inc(x_15); +x_105 = l_Lean_Syntax_node2(x_15, x_104, x_95, x_95); +x_106 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__18; +lean_inc(x_95); +lean_inc(x_15); +x_107 = l_Lean_Syntax_node3(x_15, x_106, x_5, x_105, x_95); +x_108 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__16; +lean_inc(x_15); +x_109 = l_Lean_Syntax_node1(x_15, x_108, x_107); +x_110 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__4; +lean_inc(x_15); +x_111 = l_Lean_Syntax_node5(x_15, x_110, x_88, x_97, x_103, x_109, x_95); +x_112 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__2; +x_113 = l_Lean_Syntax_node2(x_15, x_112, x_6, x_111); +if (lean_is_scalar(x_84)) { + x_114 = lean_alloc_ctor(0, 2, 0); +} else { + x_114 = x_84; +} +lean_ctor_set(x_114, 0, x_113); +lean_ctor_set(x_114, 1, x_83); +return x_114; +} +} +else +{ +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; uint8_t x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; +x_115 = lean_ctor_get(x_10, 0); +x_116 = lean_ctor_get(x_10, 1); +lean_inc(x_116); +lean_inc(x_115); +lean_dec(x_10); +x_117 = 0; +x_118 = l_Lean_SourceInfo_fromRef(x_115, x_117); +lean_dec(x_115); +x_119 = l_Lean_Elab_Command_getCurrMacroScope(x_7, x_8, x_116); +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 = l_Lean_Elab_Command_getMainModule___rarg(x_8, 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_122); + x_124 = lean_box(0); +} +x_125 = 1; +x_126 = l_Lean_SourceInfo_fromRef(x_1, x_125); +x_127 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__5; +if (lean_is_scalar(x_121)) { + x_128 = lean_alloc_ctor(2, 2, 0); +} else { + x_128 = x_121; + lean_ctor_set_tag(x_128, 2); +} +lean_ctor_set(x_128, 0, x_126); +lean_ctor_set(x_128, 1, x_127); +x_129 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__9; +x_130 = l_Lean_Name_append(x_129, x_2); +x_131 = l_Lean_Name_append(x_130, x_3); +x_132 = lean_mk_syntax_ident(x_131); +x_133 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2; +x_134 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; +lean_inc(x_118); +x_135 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_135, 0, x_118); +lean_ctor_set(x_135, 1, x_133); +lean_ctor_set(x_135, 2, x_134); +x_136 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__7; +lean_inc(x_135); +lean_inc(x_118); +x_137 = l_Lean_Syntax_node2(x_118, x_136, x_132, x_135); +x_138 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__14; +lean_inc(x_118); +x_139 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_139, 0, x_118); +lean_ctor_set(x_139, 1, x_138); +x_140 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__13; +lean_inc(x_118); +x_141 = l_Lean_Syntax_node2(x_118, x_140, x_139, x_4); +lean_inc(x_118); +x_142 = l_Lean_Syntax_node1(x_118, x_133, x_141); +x_143 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__11; +lean_inc(x_135); +lean_inc(x_118); +x_144 = l_Lean_Syntax_node2(x_118, x_143, x_135, x_142); +x_145 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__21; +lean_inc_n(x_135, 2); +lean_inc(x_118); +x_146 = l_Lean_Syntax_node2(x_118, x_145, x_135, x_135); +x_147 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__18; +lean_inc(x_135); +lean_inc(x_118); +x_148 = l_Lean_Syntax_node3(x_118, x_147, x_5, x_146, x_135); +x_149 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__16; +lean_inc(x_118); +x_150 = l_Lean_Syntax_node1(x_118, x_149, x_148); +x_151 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__4; +lean_inc(x_118); +x_152 = l_Lean_Syntax_node5(x_118, x_151, x_128, x_137, x_144, x_150, x_135); +x_153 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__2; +x_154 = l_Lean_Syntax_node2(x_118, x_153, x_6, x_152); +if (lean_is_scalar(x_124)) { + x_155 = lean_alloc_ctor(0, 2, 0); +} else { + x_155 = x_124; +} +lean_ctor_set(x_155, 0, x_154); +lean_ctor_set(x_155, 1, x_123); +return x_155; +} +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("unsupported modifiers for computed field", 40, 40); +return x_1; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___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_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__2; +x_2 = l_Lean_MessageData_ofFormat(x_1); +return x_2; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("noncomputable", 13, 13); +return x_1; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; +x_2 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__1; +x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__7; +x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; +x_2 = l_Array_append___rarg(x_1, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_11 = lean_unsigned_to_nat(4u); +x_12 = l_Lean_Syntax_getArg(x_1, x_11); +x_13 = lean_unsigned_to_nat(0u); +x_14 = l_Lean_Syntax_matchesNull(x_12, x_13); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t 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; uint8_t x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_15 = l_Lean_Elab_Command_getRef(x_8, x_9, x_10); +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_replaceRef(x_1, x_16); +lean_dec(x_16); +x_19 = lean_ctor_get(x_8, 0); +lean_inc(x_19); +x_20 = lean_ctor_get(x_8, 1); +lean_inc(x_20); +x_21 = lean_ctor_get(x_8, 2); +lean_inc(x_21); +x_22 = lean_ctor_get(x_8, 3); +lean_inc(x_22); +x_23 = lean_ctor_get(x_8, 4); +lean_inc(x_23); +x_24 = lean_ctor_get(x_8, 5); +lean_inc(x_24); +x_25 = lean_ctor_get(x_8, 7); +lean_inc(x_25); +x_26 = lean_ctor_get(x_8, 8); +lean_inc(x_26); +x_27 = lean_ctor_get(x_8, 9); +lean_inc(x_27); +x_28 = lean_ctor_get_uint8(x_8, sizeof(void*)*10); +x_29 = lean_alloc_ctor(0, 10, 1); +lean_ctor_set(x_29, 0, x_19); +lean_ctor_set(x_29, 1, x_20); +lean_ctor_set(x_29, 2, x_21); +lean_ctor_set(x_29, 3, x_22); +lean_ctor_set(x_29, 4, x_23); +lean_ctor_set(x_29, 5, x_24); +lean_ctor_set(x_29, 6, x_18); +lean_ctor_set(x_29, 7, x_25); +lean_ctor_set(x_29, 8, x_26); +lean_ctor_set(x_29, 9, x_27); +lean_ctor_set_uint8(x_29, sizeof(void*)*10, 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; +x_32 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_30, x_31, x_29, x_9, x_17); +x_33 = lean_ctor_get(x_32, 1); +lean_inc(x_33); +lean_dec(x_32); +x_34 = l_Lean_Elab_Command_getRef(x_8, x_9, x_33); +x_35 = lean_ctor_get(x_34, 0); +lean_inc(x_35); +x_36 = lean_ctor_get(x_34, 1); +lean_inc(x_36); +lean_dec(x_34); +x_37 = 0; +x_38 = l_Lean_SourceInfo_fromRef(x_35, x_37); +lean_dec(x_35); +x_39 = l_Lean_Elab_Command_getCurrMacroScope(x_8, x_9, x_36); +x_40 = lean_ctor_get(x_39, 1); +lean_inc(x_40); +lean_dec(x_39); +x_41 = l_Lean_Elab_Command_getMainModule___rarg(x_9, x_40); +x_42 = !lean_is_exclusive(x_41); +if (x_42 == 0) +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_43 = lean_ctor_get(x_41, 1); +x_44 = lean_ctor_get(x_41, 0); +lean_dec(x_44); +x_45 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2; +x_46 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; +lean_inc(x_38); +x_47 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_47, 0, x_38); +lean_ctor_set(x_47, 1, x_45); +lean_ctor_set(x_47, 2, x_46); +x_48 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; +lean_inc(x_38); +lean_ctor_set_tag(x_41, 2); +lean_ctor_set(x_41, 1, x_48); +lean_ctor_set(x_41, 0, x_38); +x_49 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; +lean_inc(x_38); +x_50 = l_Lean_Syntax_node1(x_38, x_49, x_41); +lean_inc(x_38); +x_51 = l_Lean_Syntax_node1(x_38, x_45, x_50); +lean_inc_n(x_47, 4); +x_52 = l_Lean_Syntax_node6(x_38, x_2, x_47, x_47, x_47, x_51, x_47, x_47); +x_53 = lean_apply_4(x_3, x_52, x_8, x_9, x_43); +return x_53; +} +else +{ +lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; +x_54 = lean_ctor_get(x_41, 1); +lean_inc(x_54); +lean_dec(x_41); +x_55 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2; +x_56 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; +lean_inc(x_38); +x_57 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_57, 0, x_38); +lean_ctor_set(x_57, 1, x_55); +lean_ctor_set(x_57, 2, x_56); +x_58 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; +lean_inc(x_38); +x_59 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_59, 0, x_38); +lean_ctor_set(x_59, 1, x_58); +x_60 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; +lean_inc(x_38); +x_61 = l_Lean_Syntax_node1(x_38, x_60, x_59); +lean_inc(x_38); +x_62 = l_Lean_Syntax_node1(x_38, x_55, x_61); +lean_inc_n(x_57, 4); +x_63 = l_Lean_Syntax_node6(x_38, x_2, x_57, x_57, x_57, x_62, x_57, x_57); +x_64 = lean_apply_4(x_3, x_63, x_8, x_9, x_54); +return x_64; +} +} +else +{ +lean_object* x_65; lean_object* x_66; uint8_t x_67; +x_65 = lean_unsigned_to_nat(5u); +x_66 = l_Lean_Syntax_getArg(x_1, x_65); +x_67 = l_Lean_Syntax_matchesNull(x_66, x_13); +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; 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; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; uint8_t x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; uint8_t x_95; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_68 = l_Lean_Elab_Command_getRef(x_8, x_9, x_10); +x_69 = lean_ctor_get(x_68, 0); +lean_inc(x_69); +x_70 = lean_ctor_get(x_68, 1); +lean_inc(x_70); +lean_dec(x_68); +x_71 = l_Lean_replaceRef(x_1, x_69); +lean_dec(x_69); +x_72 = lean_ctor_get(x_8, 0); +lean_inc(x_72); +x_73 = lean_ctor_get(x_8, 1); +lean_inc(x_73); +x_74 = lean_ctor_get(x_8, 2); +lean_inc(x_74); +x_75 = lean_ctor_get(x_8, 3); +lean_inc(x_75); +x_76 = lean_ctor_get(x_8, 4); +lean_inc(x_76); +x_77 = lean_ctor_get(x_8, 5); +lean_inc(x_77); +x_78 = lean_ctor_get(x_8, 7); +lean_inc(x_78); +x_79 = lean_ctor_get(x_8, 8); +lean_inc(x_79); +x_80 = lean_ctor_get(x_8, 9); +lean_inc(x_80); +x_81 = lean_ctor_get_uint8(x_8, sizeof(void*)*10); +x_82 = lean_alloc_ctor(0, 10, 1); +lean_ctor_set(x_82, 0, x_72); +lean_ctor_set(x_82, 1, x_73); +lean_ctor_set(x_82, 2, x_74); +lean_ctor_set(x_82, 3, x_75); +lean_ctor_set(x_82, 4, x_76); +lean_ctor_set(x_82, 5, x_77); +lean_ctor_set(x_82, 6, x_71); +lean_ctor_set(x_82, 7, x_78); +lean_ctor_set(x_82, 8, x_79); +lean_ctor_set(x_82, 9, x_80); +lean_ctor_set_uint8(x_82, sizeof(void*)*10, x_81); +x_83 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__3; +x_84 = 2; +x_85 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_83, x_84, x_82, x_9, x_70); +x_86 = lean_ctor_get(x_85, 1); +lean_inc(x_86); +lean_dec(x_85); +x_87 = l_Lean_Elab_Command_getRef(x_8, x_9, x_86); +x_88 = lean_ctor_get(x_87, 0); +lean_inc(x_88); +x_89 = lean_ctor_get(x_87, 1); +lean_inc(x_89); +lean_dec(x_87); +x_90 = 0; +x_91 = l_Lean_SourceInfo_fromRef(x_88, x_90); +lean_dec(x_88); +x_92 = l_Lean_Elab_Command_getCurrMacroScope(x_8, x_9, x_89); +x_93 = lean_ctor_get(x_92, 1); +lean_inc(x_93); +lean_dec(x_92); +x_94 = l_Lean_Elab_Command_getMainModule___rarg(x_9, x_93); +x_95 = !lean_is_exclusive(x_94); +if (x_95 == 0) +{ +lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; +x_96 = lean_ctor_get(x_94, 1); +x_97 = lean_ctor_get(x_94, 0); +lean_dec(x_97); +x_98 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2; +x_99 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; +lean_inc(x_91); +x_100 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_100, 0, x_91); +lean_ctor_set(x_100, 1, x_98); +lean_ctor_set(x_100, 2, x_99); +x_101 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; +lean_inc(x_91); +lean_ctor_set_tag(x_94, 2); +lean_ctor_set(x_94, 1, x_101); +lean_ctor_set(x_94, 0, x_91); +x_102 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; +lean_inc(x_91); +x_103 = l_Lean_Syntax_node1(x_91, x_102, x_94); +lean_inc(x_91); +x_104 = l_Lean_Syntax_node1(x_91, x_98, x_103); +lean_inc_n(x_100, 4); +x_105 = l_Lean_Syntax_node6(x_91, x_2, x_100, x_100, x_100, x_104, x_100, x_100); +x_106 = lean_apply_4(x_3, x_105, x_8, x_9, x_96); +return x_106; +} +else +{ +lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; +x_107 = lean_ctor_get(x_94, 1); +lean_inc(x_107); +lean_dec(x_94); +x_108 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2; +x_109 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; +lean_inc(x_91); +x_110 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_110, 0, x_91); +lean_ctor_set(x_110, 1, x_108); +lean_ctor_set(x_110, 2, x_109); +x_111 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; +lean_inc(x_91); +x_112 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_112, 0, x_91); +lean_ctor_set(x_112, 1, x_111); +x_113 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; +lean_inc(x_91); +x_114 = l_Lean_Syntax_node1(x_91, x_113, x_112); +lean_inc(x_91); +x_115 = l_Lean_Syntax_node1(x_91, x_108, x_114); +lean_inc_n(x_110, 4); +x_116 = l_Lean_Syntax_node6(x_91, x_2, x_110, x_110, x_110, x_115, x_110, x_110); +x_117 = lean_apply_4(x_3, x_116, x_8, x_9, x_107); +return x_117; +} +} +else +{ +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; uint8_t x_126; +x_118 = l_Lean_Elab_Command_getRef(x_8, x_9, x_10); +x_119 = lean_ctor_get(x_118, 0); +lean_inc(x_119); +x_120 = lean_ctor_get(x_118, 1); +lean_inc(x_120); +lean_dec(x_118); +x_121 = 0; +x_122 = l_Lean_SourceInfo_fromRef(x_119, x_121); +lean_dec(x_119); +x_123 = l_Lean_Elab_Command_getCurrMacroScope(x_8, x_9, x_120); +x_124 = lean_ctor_get(x_123, 1); +lean_inc(x_124); +lean_dec(x_123); +x_125 = l_Lean_Elab_Command_getMainModule___rarg(x_9, x_124); +x_126 = !lean_is_exclusive(x_125); +if (x_126 == 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; +x_127 = lean_ctor_get(x_125, 1); +x_128 = lean_ctor_get(x_125, 0); +lean_dec(x_128); +x_129 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; +lean_inc(x_122); +lean_ctor_set_tag(x_125, 2); +lean_ctor_set(x_125, 1, x_129); +lean_ctor_set(x_125, 0, x_122); +x_130 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; +lean_inc(x_122); +x_131 = l_Lean_Syntax_node1(x_122, x_130, x_125); +x_132 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2; +lean_inc(x_122); +x_133 = l_Lean_Syntax_node1(x_122, x_132, x_131); +x_134 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; +lean_inc(x_122); +x_135 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_135, 0, x_122); +lean_ctor_set(x_135, 1, x_132); +lean_ctor_set(x_135, 2, x_134); +if (lean_obj_tag(x_6) == 0) +{ +x_136 = x_134; +goto block_163; +} +else +{ +lean_object* x_164; lean_object* x_165; +x_164 = lean_ctor_get(x_6, 0); +lean_inc(x_164); +lean_dec(x_6); +x_165 = l_Array_mkArray1___rarg(x_164); +x_136 = x_165; +goto block_163; +} +block_163: +{ +lean_object* x_137; lean_object* x_138; +x_137 = l_Array_append___rarg(x_134, x_136); +lean_dec(x_136); +lean_inc(x_122); +x_138 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_138, 0, x_122); +lean_ctor_set(x_138, 1, x_132); +lean_ctor_set(x_138, 2, x_137); +if (lean_obj_tag(x_4) == 0) +{ +lean_object* x_139; lean_object* x_140; +x_139 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__6; +lean_inc(x_122); +x_140 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_140, 0, x_122); +lean_ctor_set(x_140, 1, x_132); +lean_ctor_set(x_140, 2, x_139); +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_141; lean_object* x_142; +lean_inc(x_135); +lean_inc(x_140); +x_141 = l_Lean_Syntax_node6(x_122, x_2, x_138, x_140, x_140, x_133, x_135, x_135); +x_142 = lean_apply_4(x_3, x_141, x_8, x_9, x_127); +return x_142; +} +else +{ +lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; +x_143 = lean_ctor_get(x_5, 0); +lean_inc(x_143); +lean_dec(x_5); +x_144 = l_Array_mkArray1___rarg(x_143); +x_145 = l_Array_append___rarg(x_134, x_144); +lean_dec(x_144); +lean_inc(x_122); +x_146 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_146, 0, x_122); +lean_ctor_set(x_146, 1, x_132); +lean_ctor_set(x_146, 2, x_145); +lean_inc(x_135); +x_147 = l_Lean_Syntax_node6(x_122, x_2, x_138, x_140, x_146, x_133, x_135, x_135); +x_148 = lean_apply_4(x_3, x_147, x_8, x_9, x_127); +return x_148; +} +} +else +{ +lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; +x_149 = lean_ctor_get(x_4, 0); +lean_inc(x_149); +lean_dec(x_4); +x_150 = l_Array_mkArray1___rarg(x_149); +x_151 = l_Array_append___rarg(x_134, x_150); +lean_dec(x_150); +lean_inc(x_122); +x_152 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_152, 0, x_122); +lean_ctor_set(x_152, 1, x_132); +lean_ctor_set(x_152, 2, x_151); +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; +x_153 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__6; +lean_inc(x_122); +x_154 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_154, 0, x_122); +lean_ctor_set(x_154, 1, x_132); +lean_ctor_set(x_154, 2, x_153); +lean_inc(x_135); +x_155 = l_Lean_Syntax_node6(x_122, x_2, x_138, x_152, x_154, x_133, x_135, x_135); +x_156 = lean_apply_4(x_3, x_155, x_8, x_9, x_127); +return x_156; +} +else +{ +lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; +x_157 = lean_ctor_get(x_5, 0); +lean_inc(x_157); +lean_dec(x_5); +x_158 = l_Array_mkArray1___rarg(x_157); +x_159 = l_Array_append___rarg(x_134, x_158); +lean_dec(x_158); +lean_inc(x_122); +x_160 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_160, 0, x_122); +lean_ctor_set(x_160, 1, x_132); +lean_ctor_set(x_160, 2, x_159); +lean_inc(x_135); +x_161 = l_Lean_Syntax_node6(x_122, x_2, x_138, x_152, x_160, x_133, x_135, x_135); +x_162 = lean_apply_4(x_3, x_161, x_8, x_9, x_127); +return x_162; +} +} +} +} +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; +x_166 = lean_ctor_get(x_125, 1); +lean_inc(x_166); +lean_dec(x_125); +x_167 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; +lean_inc(x_122); +x_168 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_168, 0, x_122); +lean_ctor_set(x_168, 1, x_167); +x_169 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; +lean_inc(x_122); +x_170 = l_Lean_Syntax_node1(x_122, x_169, x_168); +x_171 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2; +lean_inc(x_122); +x_172 = l_Lean_Syntax_node1(x_122, x_171, x_170); +x_173 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; +lean_inc(x_122); +x_174 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_174, 0, x_122); +lean_ctor_set(x_174, 1, x_171); +lean_ctor_set(x_174, 2, x_173); +if (lean_obj_tag(x_6) == 0) +{ +x_175 = x_173; +goto block_202; +} +else +{ +lean_object* x_203; lean_object* x_204; +x_203 = lean_ctor_get(x_6, 0); +lean_inc(x_203); +lean_dec(x_6); +x_204 = l_Array_mkArray1___rarg(x_203); +x_175 = x_204; +goto block_202; +} +block_202: +{ +lean_object* x_176; lean_object* x_177; +x_176 = l_Array_append___rarg(x_173, x_175); +lean_dec(x_175); +lean_inc(x_122); +x_177 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_177, 0, x_122); +lean_ctor_set(x_177, 1, x_171); +lean_ctor_set(x_177, 2, x_176); +if (lean_obj_tag(x_4) == 0) +{ +lean_object* x_178; lean_object* x_179; +x_178 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__6; +lean_inc(x_122); +x_179 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_179, 0, x_122); +lean_ctor_set(x_179, 1, x_171); +lean_ctor_set(x_179, 2, x_178); +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_180; lean_object* x_181; +lean_inc(x_174); +lean_inc(x_179); +x_180 = l_Lean_Syntax_node6(x_122, x_2, x_177, x_179, x_179, x_172, x_174, x_174); +x_181 = lean_apply_4(x_3, x_180, x_8, x_9, x_166); +return x_181; +} +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; +x_182 = lean_ctor_get(x_5, 0); +lean_inc(x_182); +lean_dec(x_5); +x_183 = l_Array_mkArray1___rarg(x_182); +x_184 = l_Array_append___rarg(x_173, x_183); +lean_dec(x_183); +lean_inc(x_122); +x_185 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_185, 0, x_122); +lean_ctor_set(x_185, 1, x_171); +lean_ctor_set(x_185, 2, x_184); +lean_inc(x_174); +x_186 = l_Lean_Syntax_node6(x_122, x_2, x_177, x_179, x_185, x_172, x_174, x_174); +x_187 = lean_apply_4(x_3, x_186, x_8, x_9, x_166); +return x_187; +} +} +else +{ +lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; +x_188 = lean_ctor_get(x_4, 0); +lean_inc(x_188); +lean_dec(x_4); +x_189 = l_Array_mkArray1___rarg(x_188); +x_190 = l_Array_append___rarg(x_173, x_189); +lean_dec(x_189); +lean_inc(x_122); +x_191 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_191, 0, x_122); +lean_ctor_set(x_191, 1, x_171); +lean_ctor_set(x_191, 2, x_190); +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; +x_192 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__6; +lean_inc(x_122); +x_193 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_193, 0, x_122); +lean_ctor_set(x_193, 1, x_171); +lean_ctor_set(x_193, 2, x_192); +lean_inc(x_174); +x_194 = l_Lean_Syntax_node6(x_122, x_2, x_177, x_191, x_193, x_172, x_174, x_174); +x_195 = lean_apply_4(x_3, x_194, x_8, x_9, x_166); +return x_195; +} +else +{ +lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; +x_196 = lean_ctor_get(x_5, 0); +lean_inc(x_196); +lean_dec(x_5); +x_197 = l_Array_mkArray1___rarg(x_196); +x_198 = l_Array_append___rarg(x_173, x_197); +lean_dec(x_197); +lean_inc(x_122); +x_199 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_199, 0, x_122); +lean_ctor_set(x_199, 1, x_171); +lean_ctor_set(x_199, 2, x_198); +lean_inc(x_174); +x_200 = l_Lean_Syntax_node6(x_122, x_2, x_177, x_191, x_199, x_172, x_174, x_174); +x_201 = lean_apply_4(x_3, x_200, x_8, x_9, x_166); +return x_201; +} +} +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_11 = lean_unsigned_to_nat(3u); +x_12 = l_Lean_Syntax_getArg(x_1, x_11); +x_13 = l_Lean_Syntax_isNone(x_12); +if (x_13 == 0) +{ +lean_object* x_14; uint8_t x_15; +x_14 = lean_unsigned_to_nat(1u); +lean_inc(x_12); +x_15 = l_Lean_Syntax_matchesNull(x_12, 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; uint8_t x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; uint8_t x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; +lean_dec(x_12); +lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_4); +x_16 = l_Lean_Elab_Command_getRef(x_8, x_9, x_10); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +x_19 = l_Lean_replaceRef(x_1, x_17); +lean_dec(x_17); +x_20 = lean_ctor_get(x_8, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_8, 1); +lean_inc(x_21); +x_22 = lean_ctor_get(x_8, 2); +lean_inc(x_22); +x_23 = lean_ctor_get(x_8, 3); +lean_inc(x_23); +x_24 = lean_ctor_get(x_8, 4); +lean_inc(x_24); +x_25 = lean_ctor_get(x_8, 5); +lean_inc(x_25); +x_26 = lean_ctor_get(x_8, 7); +lean_inc(x_26); +x_27 = lean_ctor_get(x_8, 8); +lean_inc(x_27); +x_28 = lean_ctor_get(x_8, 9); +lean_inc(x_28); +x_29 = lean_ctor_get_uint8(x_8, sizeof(void*)*10); +x_30 = lean_alloc_ctor(0, 10, 1); +lean_ctor_set(x_30, 0, x_20); +lean_ctor_set(x_30, 1, x_21); +lean_ctor_set(x_30, 2, x_22); +lean_ctor_set(x_30, 3, x_23); +lean_ctor_set(x_30, 4, x_24); +lean_ctor_set(x_30, 5, x_25); +lean_ctor_set(x_30, 6, x_19); +lean_ctor_set(x_30, 7, x_26); +lean_ctor_set(x_30, 8, x_27); +lean_ctor_set(x_30, 9, x_28); +lean_ctor_set_uint8(x_30, sizeof(void*)*10, x_29); +x_31 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__3; +x_32 = 2; +x_33 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_31, x_32, x_30, x_9, x_18); +x_34 = lean_ctor_get(x_33, 1); +lean_inc(x_34); +lean_dec(x_33); +x_35 = l_Lean_Elab_Command_getRef(x_8, x_9, 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 = 0; +x_39 = l_Lean_SourceInfo_fromRef(x_36, x_38); +lean_dec(x_36); +x_40 = l_Lean_Elab_Command_getCurrMacroScope(x_8, x_9, x_37); +x_41 = lean_ctor_get(x_40, 1); +lean_inc(x_41); +lean_dec(x_40); +x_42 = l_Lean_Elab_Command_getMainModule___rarg(x_9, x_41); +x_43 = !lean_is_exclusive(x_42); +if (x_43 == 0) +{ +lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_44 = lean_ctor_get(x_42, 1); +x_45 = lean_ctor_get(x_42, 0); +lean_dec(x_45); +x_46 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2; +x_47 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; +lean_inc(x_39); +x_48 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_48, 0, x_39); +lean_ctor_set(x_48, 1, x_46); +lean_ctor_set(x_48, 2, x_47); +x_49 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; +lean_inc(x_39); +lean_ctor_set_tag(x_42, 2); +lean_ctor_set(x_42, 1, x_49); +lean_ctor_set(x_42, 0, x_39); +x_50 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; +lean_inc(x_39); +x_51 = l_Lean_Syntax_node1(x_39, x_50, x_42); +lean_inc(x_39); +x_52 = l_Lean_Syntax_node1(x_39, x_46, x_51); +lean_inc_n(x_48, 4); +x_53 = l_Lean_Syntax_node6(x_39, x_2, x_48, x_48, x_48, x_52, x_48, x_48); +x_54 = lean_apply_4(x_3, x_53, x_8, x_9, x_44); +return x_54; +} +else +{ +lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_55 = lean_ctor_get(x_42, 1); +lean_inc(x_55); +lean_dec(x_42); +x_56 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2; +x_57 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; +lean_inc(x_39); +x_58 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_58, 0, x_39); +lean_ctor_set(x_58, 1, x_56); +lean_ctor_set(x_58, 2, x_57); +x_59 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; +lean_inc(x_39); +x_60 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_60, 0, x_39); +lean_ctor_set(x_60, 1, x_59); +x_61 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; +lean_inc(x_39); +x_62 = l_Lean_Syntax_node1(x_39, x_61, x_60); +lean_inc(x_39); +x_63 = l_Lean_Syntax_node1(x_39, x_56, x_62); +lean_inc_n(x_58, 4); +x_64 = l_Lean_Syntax_node6(x_39, x_2, x_58, x_58, x_58, x_63, x_58, x_58); +x_65 = lean_apply_4(x_3, x_64, x_8, x_9, x_55); +return x_65; +} +} +else +{ +lean_object* x_66; lean_object* x_67; lean_object* x_68; uint8_t x_69; +x_66 = lean_unsigned_to_nat(0u); +x_67 = l_Lean_Syntax_getArg(x_12, x_66); +lean_dec(x_12); +x_68 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; +x_69 = l_Lean_Syntax_isOfKind(x_67, 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; uint8_t x_83; lean_object* x_84; lean_object* x_85; uint8_t x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; uint8_t x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; uint8_t x_97; +lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_4); +x_70 = l_Lean_Elab_Command_getRef(x_8, x_9, x_10); +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_replaceRef(x_1, x_71); +lean_dec(x_71); +x_74 = lean_ctor_get(x_8, 0); +lean_inc(x_74); +x_75 = lean_ctor_get(x_8, 1); +lean_inc(x_75); +x_76 = lean_ctor_get(x_8, 2); +lean_inc(x_76); +x_77 = lean_ctor_get(x_8, 3); +lean_inc(x_77); +x_78 = lean_ctor_get(x_8, 4); +lean_inc(x_78); +x_79 = lean_ctor_get(x_8, 5); +lean_inc(x_79); +x_80 = lean_ctor_get(x_8, 7); +lean_inc(x_80); +x_81 = lean_ctor_get(x_8, 8); +lean_inc(x_81); +x_82 = lean_ctor_get(x_8, 9); +lean_inc(x_82); +x_83 = lean_ctor_get_uint8(x_8, sizeof(void*)*10); +x_84 = lean_alloc_ctor(0, 10, 1); +lean_ctor_set(x_84, 0, x_74); +lean_ctor_set(x_84, 1, x_75); +lean_ctor_set(x_84, 2, x_76); +lean_ctor_set(x_84, 3, x_77); +lean_ctor_set(x_84, 4, x_78); +lean_ctor_set(x_84, 5, x_79); +lean_ctor_set(x_84, 6, x_73); +lean_ctor_set(x_84, 7, x_80); +lean_ctor_set(x_84, 8, x_81); +lean_ctor_set(x_84, 9, x_82); +lean_ctor_set_uint8(x_84, sizeof(void*)*10, x_83); +x_85 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__3; +x_86 = 2; +x_87 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_85, x_86, x_84, x_9, x_72); +x_88 = lean_ctor_get(x_87, 1); +lean_inc(x_88); +lean_dec(x_87); +x_89 = l_Lean_Elab_Command_getRef(x_8, x_9, 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); +x_92 = 0; +x_93 = l_Lean_SourceInfo_fromRef(x_90, x_92); +lean_dec(x_90); +x_94 = l_Lean_Elab_Command_getCurrMacroScope(x_8, x_9, x_91); +x_95 = lean_ctor_get(x_94, 1); +lean_inc(x_95); +lean_dec(x_94); +x_96 = l_Lean_Elab_Command_getMainModule___rarg(x_9, x_95); +x_97 = !lean_is_exclusive(x_96); +if (x_97 == 0) +{ +lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; +x_98 = lean_ctor_get(x_96, 1); +x_99 = lean_ctor_get(x_96, 0); +lean_dec(x_99); +x_100 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2; +x_101 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; +lean_inc(x_93); +x_102 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_102, 0, x_93); +lean_ctor_set(x_102, 1, x_100); +lean_ctor_set(x_102, 2, x_101); +x_103 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; +lean_inc(x_93); +lean_ctor_set_tag(x_96, 2); +lean_ctor_set(x_96, 1, x_103); +lean_ctor_set(x_96, 0, x_93); +lean_inc(x_93); +x_104 = l_Lean_Syntax_node1(x_93, x_68, x_96); +lean_inc(x_93); +x_105 = l_Lean_Syntax_node1(x_93, x_100, x_104); +lean_inc_n(x_102, 4); +x_106 = l_Lean_Syntax_node6(x_93, x_2, x_102, x_102, x_102, x_105, x_102, x_102); +x_107 = lean_apply_4(x_3, x_106, x_8, x_9, x_98); +return x_107; +} +else +{ +lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; +x_108 = lean_ctor_get(x_96, 1); +lean_inc(x_108); +lean_dec(x_96); +x_109 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2; +x_110 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; +lean_inc(x_93); +x_111 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_111, 0, x_93); +lean_ctor_set(x_111, 1, x_109); +lean_ctor_set(x_111, 2, x_110); +x_112 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; +lean_inc(x_93); +x_113 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_113, 0, x_93); +lean_ctor_set(x_113, 1, x_112); +lean_inc(x_93); +x_114 = l_Lean_Syntax_node1(x_93, x_68, x_113); +lean_inc(x_93); +x_115 = l_Lean_Syntax_node1(x_93, x_109, x_114); +lean_inc_n(x_111, 4); +x_116 = l_Lean_Syntax_node6(x_93, x_2, x_111, x_111, x_111, x_115, x_111, x_111); +x_117 = lean_apply_4(x_3, x_116, x_8, x_9, x_108); +return x_117; +} +} +else +{ +lean_object* x_118; lean_object* x_119; +x_118 = lean_box(0); +x_119 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2(x_1, x_2, x_3, x_4, x_7, x_5, x_118, x_8, x_9, x_10); +return x_119; +} +} +} +else +{ +lean_object* x_120; lean_object* x_121; +lean_dec(x_12); +x_120 = lean_box(0); +x_121 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2(x_1, x_2, x_3, x_4, x_7, x_5, x_120, x_8, x_9, x_10); +return x_121; +} +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; uint8_t x_12; +x_10 = lean_unsigned_to_nat(2u); +x_11 = l_Lean_Syntax_getArg(x_1, x_10); +x_12 = l_Lean_Syntax_isNone(x_11); +if (x_12 == 0) +{ +lean_object* x_13; uint8_t x_14; +x_13 = lean_unsigned_to_nat(1u); +lean_inc(x_11); +x_14 = l_Lean_Syntax_matchesNull(x_11, x_13); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t 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; uint8_t x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; +lean_dec(x_11); +lean_dec(x_6); +lean_dec(x_4); +x_15 = l_Lean_Elab_Command_getRef(x_7, x_8, x_9); +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_replaceRef(x_1, x_16); +lean_dec(x_16); +x_19 = lean_ctor_get(x_7, 0); +lean_inc(x_19); +x_20 = lean_ctor_get(x_7, 1); +lean_inc(x_20); +x_21 = lean_ctor_get(x_7, 2); +lean_inc(x_21); +x_22 = lean_ctor_get(x_7, 3); +lean_inc(x_22); +x_23 = lean_ctor_get(x_7, 4); +lean_inc(x_23); +x_24 = lean_ctor_get(x_7, 5); +lean_inc(x_24); +x_25 = lean_ctor_get(x_7, 7); +lean_inc(x_25); +x_26 = lean_ctor_get(x_7, 8); +lean_inc(x_26); +x_27 = lean_ctor_get(x_7, 9); +lean_inc(x_27); +x_28 = lean_ctor_get_uint8(x_7, sizeof(void*)*10); +x_29 = lean_alloc_ctor(0, 10, 1); +lean_ctor_set(x_29, 0, x_19); +lean_ctor_set(x_29, 1, x_20); +lean_ctor_set(x_29, 2, x_21); +lean_ctor_set(x_29, 3, x_22); +lean_ctor_set(x_29, 4, x_23); +lean_ctor_set(x_29, 5, x_24); +lean_ctor_set(x_29, 6, x_18); +lean_ctor_set(x_29, 7, x_25); +lean_ctor_set(x_29, 8, x_26); +lean_ctor_set(x_29, 9, x_27); +lean_ctor_set_uint8(x_29, sizeof(void*)*10, 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; +x_32 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_30, x_31, x_29, x_8, x_17); +x_33 = lean_ctor_get(x_32, 1); +lean_inc(x_33); +lean_dec(x_32); +x_34 = l_Lean_Elab_Command_getRef(x_7, x_8, x_33); +x_35 = lean_ctor_get(x_34, 0); +lean_inc(x_35); +x_36 = lean_ctor_get(x_34, 1); +lean_inc(x_36); +lean_dec(x_34); +x_37 = 0; +x_38 = l_Lean_SourceInfo_fromRef(x_35, x_37); +lean_dec(x_35); +x_39 = l_Lean_Elab_Command_getCurrMacroScope(x_7, x_8, x_36); +x_40 = lean_ctor_get(x_39, 1); +lean_inc(x_40); +lean_dec(x_39); +x_41 = l_Lean_Elab_Command_getMainModule___rarg(x_8, x_40); +x_42 = !lean_is_exclusive(x_41); +if (x_42 == 0) +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_43 = lean_ctor_get(x_41, 1); +x_44 = lean_ctor_get(x_41, 0); +lean_dec(x_44); +x_45 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2; +x_46 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; +lean_inc(x_38); +x_47 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_47, 0, x_38); +lean_ctor_set(x_47, 1, x_45); +lean_ctor_set(x_47, 2, x_46); +x_48 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; +lean_inc(x_38); +lean_ctor_set_tag(x_41, 2); +lean_ctor_set(x_41, 1, x_48); +lean_ctor_set(x_41, 0, x_38); +x_49 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; +lean_inc(x_38); +x_50 = l_Lean_Syntax_node1(x_38, x_49, x_41); +lean_inc(x_38); +x_51 = l_Lean_Syntax_node1(x_38, x_45, x_50); +lean_inc_n(x_47, 4); +x_52 = l_Lean_Syntax_node6(x_38, x_2, x_47, x_47, x_47, x_51, x_47, x_47); +x_53 = lean_apply_4(x_3, x_52, x_7, x_8, x_43); +return x_53; +} +else +{ +lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; +x_54 = lean_ctor_get(x_41, 1); +lean_inc(x_54); +lean_dec(x_41); +x_55 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2; +x_56 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; +lean_inc(x_38); +x_57 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_57, 0, x_38); +lean_ctor_set(x_57, 1, x_55); +lean_ctor_set(x_57, 2, x_56); +x_58 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; +lean_inc(x_38); +x_59 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_59, 0, x_38); +lean_ctor_set(x_59, 1, x_58); +x_60 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; +lean_inc(x_38); +x_61 = l_Lean_Syntax_node1(x_38, x_60, x_59); +lean_inc(x_38); +x_62 = l_Lean_Syntax_node1(x_38, x_55, x_61); +lean_inc_n(x_57, 4); +x_63 = l_Lean_Syntax_node6(x_38, x_2, x_57, x_57, x_57, x_62, x_57, x_57); +x_64 = lean_apply_4(x_3, x_63, x_7, x_8, x_54); +return x_64; +} +} +else +{ +lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; +x_65 = lean_unsigned_to_nat(0u); +x_66 = l_Lean_Syntax_getArg(x_11, x_65); +lean_dec(x_11); +x_67 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_67, 0, x_66); +x_68 = lean_box(0); +x_69 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__3(x_1, x_2, x_3, x_6, x_4, x_68, x_67, x_7, x_8, x_9); +return x_69; +} +} +else +{ +lean_object* x_70; lean_object* x_71; lean_object* x_72; +lean_dec(x_11); +x_70 = lean_box(0); +x_71 = lean_box(0); +x_72 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__3(x_1, x_2, x_3, x_6, x_4, x_71, x_70, x_7, x_8, x_9); +return x_72; +} +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__5___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("attributes", 10, 10); +return x_1; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__5___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; +x_2 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__1; +x_3 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__1___closed__1; +x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__5___closed__1; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___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; uint8_t x_11; +x_9 = lean_unsigned_to_nat(1u); +x_10 = l_Lean_Syntax_getArg(x_1, x_9); +x_11 = l_Lean_Syntax_isNone(x_10); +if (x_11 == 0) +{ +uint8_t x_12; +lean_inc(x_10); +x_12 = l_Lean_Syntax_matchesNull(x_10, x_9); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; 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; uint8_t x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; +lean_dec(x_10); +lean_dec(x_5); +x_13 = l_Lean_Elab_Command_getRef(x_6, x_7, x_8); +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_replaceRef(x_1, x_14); +lean_dec(x_14); +x_17 = lean_ctor_get(x_6, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_6, 1); +lean_inc(x_18); +x_19 = lean_ctor_get(x_6, 2); +lean_inc(x_19); +x_20 = lean_ctor_get(x_6, 3); +lean_inc(x_20); +x_21 = lean_ctor_get(x_6, 4); +lean_inc(x_21); +x_22 = lean_ctor_get(x_6, 5); +lean_inc(x_22); +x_23 = lean_ctor_get(x_6, 7); +lean_inc(x_23); +x_24 = lean_ctor_get(x_6, 8); +lean_inc(x_24); +x_25 = lean_ctor_get(x_6, 9); +lean_inc(x_25); +x_26 = lean_ctor_get_uint8(x_6, sizeof(void*)*10); +x_27 = lean_alloc_ctor(0, 10, 1); +lean_ctor_set(x_27, 0, x_17); +lean_ctor_set(x_27, 1, x_18); +lean_ctor_set(x_27, 2, x_19); +lean_ctor_set(x_27, 3, x_20); +lean_ctor_set(x_27, 4, x_21); +lean_ctor_set(x_27, 5, x_22); +lean_ctor_set(x_27, 6, x_16); +lean_ctor_set(x_27, 7, x_23); +lean_ctor_set(x_27, 8, x_24); +lean_ctor_set(x_27, 9, x_25); +lean_ctor_set_uint8(x_27, sizeof(void*)*10, 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; +x_30 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_28, x_29, x_27, x_7, x_15); +x_31 = lean_ctor_get(x_30, 1); +lean_inc(x_31); +lean_dec(x_30); +x_32 = l_Lean_Elab_Command_getRef(x_6, x_7, 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); +lean_dec(x_32); +x_35 = 0; +x_36 = l_Lean_SourceInfo_fromRef(x_33, x_35); +lean_dec(x_33); +x_37 = l_Lean_Elab_Command_getCurrMacroScope(x_6, x_7, x_34); +x_38 = lean_ctor_get(x_37, 1); +lean_inc(x_38); +lean_dec(x_37); +x_39 = l_Lean_Elab_Command_getMainModule___rarg(x_7, x_38); +x_40 = !lean_is_exclusive(x_39); +if (x_40 == 0) +{ +lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_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_39, 1); +x_42 = lean_ctor_get(x_39, 0); +lean_dec(x_42); +x_43 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2; +x_44 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; +lean_inc(x_36); +x_45 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_45, 0, x_36); +lean_ctor_set(x_45, 1, x_43); +lean_ctor_set(x_45, 2, x_44); +x_46 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; +lean_inc(x_36); +lean_ctor_set_tag(x_39, 2); +lean_ctor_set(x_39, 1, x_46); +lean_ctor_set(x_39, 0, x_36); +x_47 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; +lean_inc(x_36); +x_48 = l_Lean_Syntax_node1(x_36, x_47, x_39); +lean_inc(x_36); +x_49 = l_Lean_Syntax_node1(x_36, x_43, x_48); +lean_inc_n(x_45, 4); +x_50 = l_Lean_Syntax_node6(x_36, x_2, x_45, x_45, x_45, x_49, x_45, x_45); +x_51 = lean_apply_4(x_3, x_50, x_6, x_7, x_41); +return x_51; +} +else +{ +lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; +x_52 = lean_ctor_get(x_39, 1); +lean_inc(x_52); +lean_dec(x_39); +x_53 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2; +x_54 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; +lean_inc(x_36); +x_55 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_55, 0, x_36); +lean_ctor_set(x_55, 1, x_53); +lean_ctor_set(x_55, 2, x_54); +x_56 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; +lean_inc(x_36); +x_57 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_57, 0, x_36); +lean_ctor_set(x_57, 1, x_56); +x_58 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; +lean_inc(x_36); +x_59 = l_Lean_Syntax_node1(x_36, x_58, x_57); +lean_inc(x_36); +x_60 = l_Lean_Syntax_node1(x_36, x_53, x_59); +lean_inc_n(x_55, 4); +x_61 = l_Lean_Syntax_node6(x_36, x_2, x_55, x_55, x_55, x_60, x_55, x_55); +x_62 = lean_apply_4(x_3, x_61, x_6, x_7, x_52); +return x_62; +} +} +else +{ +lean_object* x_63; lean_object* x_64; lean_object* x_65; uint8_t x_66; +x_63 = lean_unsigned_to_nat(0u); +x_64 = l_Lean_Syntax_getArg(x_10, x_63); +lean_dec(x_10); +x_65 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__5___closed__2; +lean_inc(x_64); +x_66 = l_Lean_Syntax_isOfKind(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; lean_object* x_78; lean_object* x_79; uint8_t x_80; lean_object* x_81; lean_object* x_82; uint8_t x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; uint8_t x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; uint8_t x_94; +lean_dec(x_64); +lean_dec(x_5); +x_67 = l_Lean_Elab_Command_getRef(x_6, x_7, x_8); +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 = l_Lean_replaceRef(x_1, x_68); +lean_dec(x_68); +x_71 = lean_ctor_get(x_6, 0); +lean_inc(x_71); +x_72 = lean_ctor_get(x_6, 1); +lean_inc(x_72); +x_73 = lean_ctor_get(x_6, 2); +lean_inc(x_73); +x_74 = lean_ctor_get(x_6, 3); +lean_inc(x_74); +x_75 = lean_ctor_get(x_6, 4); +lean_inc(x_75); +x_76 = lean_ctor_get(x_6, 5); +lean_inc(x_76); +x_77 = lean_ctor_get(x_6, 7); +lean_inc(x_77); +x_78 = lean_ctor_get(x_6, 8); +lean_inc(x_78); +x_79 = lean_ctor_get(x_6, 9); +lean_inc(x_79); +x_80 = lean_ctor_get_uint8(x_6, sizeof(void*)*10); +x_81 = lean_alloc_ctor(0, 10, 1); +lean_ctor_set(x_81, 0, x_71); +lean_ctor_set(x_81, 1, x_72); +lean_ctor_set(x_81, 2, x_73); +lean_ctor_set(x_81, 3, x_74); +lean_ctor_set(x_81, 4, x_75); +lean_ctor_set(x_81, 5, x_76); +lean_ctor_set(x_81, 6, x_70); +lean_ctor_set(x_81, 7, x_77); +lean_ctor_set(x_81, 8, x_78); +lean_ctor_set(x_81, 9, x_79); +lean_ctor_set_uint8(x_81, sizeof(void*)*10, x_80); +x_82 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__3; +x_83 = 2; +x_84 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_82, x_83, x_81, x_7, x_69); +x_85 = lean_ctor_get(x_84, 1); +lean_inc(x_85); +lean_dec(x_84); +x_86 = l_Lean_Elab_Command_getRef(x_6, x_7, x_85); +x_87 = lean_ctor_get(x_86, 0); +lean_inc(x_87); +x_88 = lean_ctor_get(x_86, 1); +lean_inc(x_88); +lean_dec(x_86); +x_89 = 0; +x_90 = l_Lean_SourceInfo_fromRef(x_87, x_89); +lean_dec(x_87); +x_91 = l_Lean_Elab_Command_getCurrMacroScope(x_6, x_7, x_88); +x_92 = lean_ctor_get(x_91, 1); +lean_inc(x_92); +lean_dec(x_91); +x_93 = l_Lean_Elab_Command_getMainModule___rarg(x_7, x_92); +x_94 = !lean_is_exclusive(x_93); +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_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; +x_95 = lean_ctor_get(x_93, 1); +x_96 = lean_ctor_get(x_93, 0); +lean_dec(x_96); +x_97 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2; +x_98 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; +lean_inc(x_90); +x_99 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_99, 0, x_90); +lean_ctor_set(x_99, 1, x_97); +lean_ctor_set(x_99, 2, x_98); +x_100 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; +lean_inc(x_90); +lean_ctor_set_tag(x_93, 2); +lean_ctor_set(x_93, 1, x_100); +lean_ctor_set(x_93, 0, x_90); +x_101 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; +lean_inc(x_90); +x_102 = l_Lean_Syntax_node1(x_90, x_101, x_93); +lean_inc(x_90); +x_103 = l_Lean_Syntax_node1(x_90, x_97, x_102); +lean_inc_n(x_99, 4); +x_104 = l_Lean_Syntax_node6(x_90, x_2, x_99, x_99, x_99, x_103, x_99, x_99); +x_105 = lean_apply_4(x_3, x_104, x_6, x_7, x_95); +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; lean_object* x_114; lean_object* x_115; lean_object* x_116; +x_106 = lean_ctor_get(x_93, 1); +lean_inc(x_106); +lean_dec(x_93); +x_107 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2; +x_108 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; +lean_inc(x_90); +x_109 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_109, 0, x_90); +lean_ctor_set(x_109, 1, x_107); +lean_ctor_set(x_109, 2, x_108); +x_110 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; +lean_inc(x_90); +x_111 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_111, 0, x_90); +lean_ctor_set(x_111, 1, x_110); +x_112 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; +lean_inc(x_90); +x_113 = l_Lean_Syntax_node1(x_90, x_112, x_111); +lean_inc(x_90); +x_114 = l_Lean_Syntax_node1(x_90, x_107, x_113); +lean_inc_n(x_109, 4); +x_115 = l_Lean_Syntax_node6(x_90, x_2, x_109, x_109, x_109, x_114, x_109, x_109); +x_116 = lean_apply_4(x_3, x_115, x_6, x_7, x_106); +return x_116; +} +} +else +{ +lean_object* x_117; lean_object* x_118; lean_object* x_119; +x_117 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_117, 0, x_64); +x_118 = lean_box(0); +x_119 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__4(x_1, x_2, x_3, x_5, x_118, x_117, x_6, x_7, x_8); +return x_119; +} +} +} +else +{ +lean_object* x_120; lean_object* x_121; lean_object* x_122; +lean_dec(x_10); +x_120 = lean_box(0); +x_121 = lean_box(0); +x_122 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__4(x_1, x_2, x_3, x_5, x_121, x_120, x_6, x_7, x_8); +return x_122; +} +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("declModifiers", 13, 13); +return x_1; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; +x_2 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__1; +x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__7; +x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___closed__1; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("docComment", 10, 10); +return x_1; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; +x_2 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__1; +x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__7; +x_4 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___closed__3; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___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) { +_start: +{ +uint8_t x_9; +x_9 = lean_usize_dec_lt(x_4, x_3); +if (x_9 == 0) +{ +lean_object* x_10; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_1); +x_10 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_10, 0, x_5); +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_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; uint8_t x_27; +x_11 = lean_array_uget(x_2, x_4); +x_19 = lean_ctor_get(x_11, 0); +lean_inc(x_19); +x_20 = lean_ctor_get(x_11, 1); +lean_inc(x_20); +x_21 = lean_ctor_get(x_11, 2); +lean_inc(x_21); +x_22 = lean_ctor_get(x_11, 3); +lean_inc(x_22); +x_23 = lean_ctor_get(x_11, 4); +lean_inc(x_23); +lean_dec(x_11); +lean_inc(x_23); +lean_inc(x_22); +lean_inc(x_21); +lean_inc(x_1); +lean_inc(x_19); +x_24 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___boxed), 9, 5); +lean_closure_set(x_24, 0, x_19); +lean_closure_set(x_24, 1, x_1); +lean_closure_set(x_24, 2, x_21); +lean_closure_set(x_24, 3, x_22); +lean_closure_set(x_24, 4, x_23); +x_25 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___closed__2; +lean_inc(x_20); +x_26 = l_Lean_Syntax_isOfKind(x_20, x_25); +if (x_26 == 0) +{ +uint8_t x_217; +x_217 = 0; +x_27 = x_217; +goto block_216; +} +else +{ +uint8_t x_218; +x_218 = 1; +x_27 = x_218; +goto block_216; +} +block_18: +{ +lean_object* x_14; size_t x_15; size_t x_16; +x_14 = lean_array_push(x_5, x_12); +x_15 = 1; +x_16 = lean_usize_add(x_4, x_15); +x_4 = x_16; +x_5 = x_14; +x_8 = x_13; +goto _start; +} +block_216: +{ +if (x_27 == 0) +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; uint8_t 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_24); +x_28 = l_Lean_Elab_Command_getRef(x_6, x_7, x_8); +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_replaceRef(x_20, x_29); +lean_dec(x_29); +lean_dec(x_20); +x_32 = lean_ctor_get(x_6, 0); +lean_inc(x_32); +x_33 = lean_ctor_get(x_6, 1); +lean_inc(x_33); +x_34 = lean_ctor_get(x_6, 2); +lean_inc(x_34); +x_35 = lean_ctor_get(x_6, 3); +lean_inc(x_35); +x_36 = lean_ctor_get(x_6, 4); +lean_inc(x_36); +x_37 = lean_ctor_get(x_6, 5); +lean_inc(x_37); +x_38 = lean_ctor_get(x_6, 7); +lean_inc(x_38); +x_39 = lean_ctor_get(x_6, 8); +lean_inc(x_39); +x_40 = lean_ctor_get(x_6, 9); +lean_inc(x_40); +x_41 = lean_ctor_get_uint8(x_6, sizeof(void*)*10); +x_42 = lean_alloc_ctor(0, 10, 1); +lean_ctor_set(x_42, 0, x_32); +lean_ctor_set(x_42, 1, x_33); +lean_ctor_set(x_42, 2, x_34); +lean_ctor_set(x_42, 3, x_35); +lean_ctor_set(x_42, 4, x_36); +lean_ctor_set(x_42, 5, x_37); +lean_ctor_set(x_42, 6, x_31); +lean_ctor_set(x_42, 7, x_38); +lean_ctor_set(x_42, 8, x_39); +lean_ctor_set(x_42, 9, x_40); +lean_ctor_set_uint8(x_42, sizeof(void*)*10, x_41); +x_43 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__3; +x_44 = 2; +x_45 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_43, x_44, x_42, x_7, x_30); +x_46 = lean_ctor_get(x_45, 1); +lean_inc(x_46); +lean_dec(x_45); +x_47 = l_Lean_Elab_Command_getRef(x_6, x_7, x_46); +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 = 0; +x_51 = l_Lean_SourceInfo_fromRef(x_48, x_50); +lean_dec(x_48); +x_52 = l_Lean_Elab_Command_getCurrMacroScope(x_6, x_7, x_49); +x_53 = lean_ctor_get(x_52, 1); +lean_inc(x_53); +lean_dec(x_52); +x_54 = l_Lean_Elab_Command_getMainModule___rarg(x_7, x_53); +x_55 = !lean_is_exclusive(x_54); +if (x_55 == 0) +{ +lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; 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_56 = lean_ctor_get(x_54, 1); +x_57 = lean_ctor_get(x_54, 0); +lean_dec(x_57); +x_58 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2; +x_59 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; +lean_inc(x_51); +x_60 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_60, 0, x_51); +lean_ctor_set(x_60, 1, x_58); +lean_ctor_set(x_60, 2, x_59); +x_61 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; +lean_inc(x_51); +lean_ctor_set_tag(x_54, 2); +lean_ctor_set(x_54, 1, x_61); +lean_ctor_set(x_54, 0, x_51); +x_62 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; +lean_inc(x_51); +x_63 = l_Lean_Syntax_node1(x_51, x_62, x_54); +lean_inc(x_51); +x_64 = l_Lean_Syntax_node1(x_51, x_58, x_63); +lean_inc_n(x_60, 4); +x_65 = l_Lean_Syntax_node6(x_51, x_25, x_60, x_60, x_60, x_64, x_60, x_60); +lean_inc(x_1); +x_66 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1(x_19, x_1, x_21, x_22, x_23, x_65, x_6, x_7, x_56); +lean_dec(x_19); +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_12 = x_67; +x_13 = x_68; +goto block_18; +} +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_54, 1); +lean_inc(x_69); +lean_dec(x_54); +x_70 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2; +x_71 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; +lean_inc(x_51); +x_72 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_72, 0, x_51); +lean_ctor_set(x_72, 1, x_70); +lean_ctor_set(x_72, 2, x_71); +x_73 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; +lean_inc(x_51); +x_74 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_74, 0, x_51); +lean_ctor_set(x_74, 1, x_73); +x_75 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; +lean_inc(x_51); +x_76 = l_Lean_Syntax_node1(x_51, x_75, x_74); +lean_inc(x_51); +x_77 = l_Lean_Syntax_node1(x_51, x_70, x_76); +lean_inc_n(x_72, 4); +x_78 = l_Lean_Syntax_node6(x_51, x_25, x_72, x_72, x_72, x_77, x_72, x_72); +lean_inc(x_1); +x_79 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1(x_19, x_1, x_21, x_22, x_23, x_78, x_6, x_7, x_69); +lean_dec(x_19); +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_12 = x_80; +x_13 = x_81; +goto block_18; +} +} +else +{ +lean_object* x_82; lean_object* x_83; uint8_t x_84; +x_82 = lean_unsigned_to_nat(0u); +x_83 = l_Lean_Syntax_getArg(x_20, x_82); +x_84 = l_Lean_Syntax_isNone(x_83); +if (x_84 == 0) +{ +lean_object* x_85; uint8_t x_86; +x_85 = lean_unsigned_to_nat(1u); +lean_inc(x_83); +x_86 = l_Lean_Syntax_matchesNull(x_83, x_85); +if (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_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; uint8_t x_100; lean_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; uint8_t x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; uint8_t x_114; +lean_dec(x_83); +lean_dec(x_24); +x_87 = l_Lean_Elab_Command_getRef(x_6, x_7, x_8); +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); +x_90 = l_Lean_replaceRef(x_20, x_88); +lean_dec(x_88); +lean_dec(x_20); +x_91 = lean_ctor_get(x_6, 0); +lean_inc(x_91); +x_92 = lean_ctor_get(x_6, 1); +lean_inc(x_92); +x_93 = lean_ctor_get(x_6, 2); +lean_inc(x_93); +x_94 = lean_ctor_get(x_6, 3); +lean_inc(x_94); +x_95 = lean_ctor_get(x_6, 4); +lean_inc(x_95); +x_96 = lean_ctor_get(x_6, 5); +lean_inc(x_96); +x_97 = lean_ctor_get(x_6, 7); +lean_inc(x_97); +x_98 = lean_ctor_get(x_6, 8); +lean_inc(x_98); +x_99 = lean_ctor_get(x_6, 9); +lean_inc(x_99); +x_100 = lean_ctor_get_uint8(x_6, sizeof(void*)*10); +x_101 = lean_alloc_ctor(0, 10, 1); +lean_ctor_set(x_101, 0, x_91); +lean_ctor_set(x_101, 1, x_92); +lean_ctor_set(x_101, 2, x_93); +lean_ctor_set(x_101, 3, x_94); +lean_ctor_set(x_101, 4, x_95); +lean_ctor_set(x_101, 5, x_96); +lean_ctor_set(x_101, 6, x_90); +lean_ctor_set(x_101, 7, x_97); +lean_ctor_set(x_101, 8, x_98); +lean_ctor_set(x_101, 9, x_99); +lean_ctor_set_uint8(x_101, sizeof(void*)*10, x_100); +x_102 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__3; +x_103 = 2; +x_104 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_102, x_103, x_101, x_7, x_89); +x_105 = lean_ctor_get(x_104, 1); +lean_inc(x_105); +lean_dec(x_104); +x_106 = l_Lean_Elab_Command_getRef(x_6, x_7, 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 = 0; +x_110 = l_Lean_SourceInfo_fromRef(x_107, x_109); +lean_dec(x_107); +x_111 = l_Lean_Elab_Command_getCurrMacroScope(x_6, x_7, x_108); +x_112 = lean_ctor_get(x_111, 1); +lean_inc(x_112); +lean_dec(x_111); +x_113 = l_Lean_Elab_Command_getMainModule___rarg(x_7, x_112); +x_114 = !lean_is_exclusive(x_113); +if (x_114 == 0) +{ +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_115 = lean_ctor_get(x_113, 1); +x_116 = lean_ctor_get(x_113, 0); +lean_dec(x_116); +x_117 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2; +x_118 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; +lean_inc(x_110); +x_119 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_119, 0, x_110); +lean_ctor_set(x_119, 1, x_117); +lean_ctor_set(x_119, 2, x_118); +x_120 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; +lean_inc(x_110); +lean_ctor_set_tag(x_113, 2); +lean_ctor_set(x_113, 1, x_120); +lean_ctor_set(x_113, 0, x_110); +x_121 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; +lean_inc(x_110); +x_122 = l_Lean_Syntax_node1(x_110, x_121, x_113); +lean_inc(x_110); +x_123 = l_Lean_Syntax_node1(x_110, x_117, x_122); +lean_inc_n(x_119, 4); +x_124 = l_Lean_Syntax_node6(x_110, x_25, x_119, x_119, x_119, x_123, x_119, x_119); +lean_inc(x_1); +x_125 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1(x_19, x_1, x_21, x_22, x_23, x_124, x_6, x_7, x_115); +lean_dec(x_19); +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_12 = x_126; +x_13 = x_127; +goto block_18; +} +else +{ +lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; +x_128 = lean_ctor_get(x_113, 1); +lean_inc(x_128); +lean_dec(x_113); +x_129 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2; +x_130 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; +lean_inc(x_110); +x_131 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_131, 0, x_110); +lean_ctor_set(x_131, 1, x_129); +lean_ctor_set(x_131, 2, x_130); +x_132 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; +lean_inc(x_110); +x_133 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_133, 0, x_110); +lean_ctor_set(x_133, 1, x_132); +x_134 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; +lean_inc(x_110); +x_135 = l_Lean_Syntax_node1(x_110, x_134, x_133); +lean_inc(x_110); +x_136 = l_Lean_Syntax_node1(x_110, x_129, x_135); +lean_inc_n(x_131, 4); +x_137 = l_Lean_Syntax_node6(x_110, x_25, x_131, x_131, x_131, x_136, x_131, x_131); +lean_inc(x_1); +x_138 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1(x_19, x_1, x_21, x_22, x_23, x_137, x_6, x_7, x_128); +lean_dec(x_19); +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_12 = x_139; +x_13 = x_140; +goto block_18; +} +} +else +{ +lean_object* x_141; lean_object* x_142; uint8_t x_143; +x_141 = l_Lean_Syntax_getArg(x_83, x_82); +lean_dec(x_83); +x_142 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___closed__4; +lean_inc(x_141); +x_143 = l_Lean_Syntax_isOfKind(x_141, x_142); +if (x_143 == 0) +{ +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; uint8_t x_157; lean_object* x_158; lean_object* x_159; uint8_t x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; uint8_t x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; uint8_t x_171; +lean_dec(x_141); +lean_dec(x_24); +x_144 = l_Lean_Elab_Command_getRef(x_6, x_7, x_8); +x_145 = lean_ctor_get(x_144, 0); +lean_inc(x_145); +x_146 = lean_ctor_get(x_144, 1); +lean_inc(x_146); +lean_dec(x_144); +x_147 = l_Lean_replaceRef(x_20, x_145); +lean_dec(x_145); +lean_dec(x_20); +x_148 = lean_ctor_get(x_6, 0); +lean_inc(x_148); +x_149 = lean_ctor_get(x_6, 1); +lean_inc(x_149); +x_150 = lean_ctor_get(x_6, 2); +lean_inc(x_150); +x_151 = lean_ctor_get(x_6, 3); +lean_inc(x_151); +x_152 = lean_ctor_get(x_6, 4); +lean_inc(x_152); +x_153 = lean_ctor_get(x_6, 5); +lean_inc(x_153); +x_154 = lean_ctor_get(x_6, 7); +lean_inc(x_154); +x_155 = lean_ctor_get(x_6, 8); +lean_inc(x_155); +x_156 = lean_ctor_get(x_6, 9); +lean_inc(x_156); +x_157 = lean_ctor_get_uint8(x_6, sizeof(void*)*10); +x_158 = lean_alloc_ctor(0, 10, 1); +lean_ctor_set(x_158, 0, x_148); +lean_ctor_set(x_158, 1, x_149); +lean_ctor_set(x_158, 2, x_150); +lean_ctor_set(x_158, 3, x_151); +lean_ctor_set(x_158, 4, x_152); +lean_ctor_set(x_158, 5, x_153); +lean_ctor_set(x_158, 6, x_147); +lean_ctor_set(x_158, 7, x_154); +lean_ctor_set(x_158, 8, x_155); +lean_ctor_set(x_158, 9, x_156); +lean_ctor_set_uint8(x_158, sizeof(void*)*10, x_157); +x_159 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__3; +x_160 = 2; +x_161 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_159, x_160, x_158, x_7, x_146); +x_162 = lean_ctor_get(x_161, 1); +lean_inc(x_162); +lean_dec(x_161); +x_163 = l_Lean_Elab_Command_getRef(x_6, x_7, x_162); +x_164 = lean_ctor_get(x_163, 0); +lean_inc(x_164); +x_165 = lean_ctor_get(x_163, 1); +lean_inc(x_165); +lean_dec(x_163); +x_166 = 0; +x_167 = l_Lean_SourceInfo_fromRef(x_164, x_166); +lean_dec(x_164); +x_168 = l_Lean_Elab_Command_getCurrMacroScope(x_6, x_7, x_165); +x_169 = lean_ctor_get(x_168, 1); +lean_inc(x_169); +lean_dec(x_168); +x_170 = l_Lean_Elab_Command_getMainModule___rarg(x_7, x_169); +x_171 = !lean_is_exclusive(x_170); +if (x_171 == 0) +{ +lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; +x_172 = lean_ctor_get(x_170, 1); +x_173 = lean_ctor_get(x_170, 0); +lean_dec(x_173); +x_174 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2; +x_175 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; +lean_inc(x_167); +x_176 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_176, 0, x_167); +lean_ctor_set(x_176, 1, x_174); +lean_ctor_set(x_176, 2, x_175); +x_177 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; +lean_inc(x_167); +lean_ctor_set_tag(x_170, 2); +lean_ctor_set(x_170, 1, x_177); +lean_ctor_set(x_170, 0, x_167); +x_178 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; +lean_inc(x_167); +x_179 = l_Lean_Syntax_node1(x_167, x_178, x_170); +lean_inc(x_167); +x_180 = l_Lean_Syntax_node1(x_167, x_174, x_179); +lean_inc_n(x_176, 4); +x_181 = l_Lean_Syntax_node6(x_167, x_25, x_176, x_176, x_176, x_180, x_176, x_176); +lean_inc(x_1); +x_182 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1(x_19, x_1, x_21, x_22, x_23, x_181, x_6, x_7, x_172); +lean_dec(x_19); +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_12 = x_183; +x_13 = x_184; +goto block_18; +} +else +{ +lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; 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_185 = lean_ctor_get(x_170, 1); +lean_inc(x_185); +lean_dec(x_170); +x_186 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2; +x_187 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; +lean_inc(x_167); +x_188 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_188, 0, x_167); +lean_ctor_set(x_188, 1, x_186); +lean_ctor_set(x_188, 2, x_187); +x_189 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; +lean_inc(x_167); +x_190 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_190, 0, x_167); +lean_ctor_set(x_190, 1, x_189); +x_191 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; +lean_inc(x_167); +x_192 = l_Lean_Syntax_node1(x_167, x_191, x_190); +lean_inc(x_167); +x_193 = l_Lean_Syntax_node1(x_167, x_186, x_192); +lean_inc_n(x_188, 4); +x_194 = l_Lean_Syntax_node6(x_167, x_25, x_188, x_188, x_188, x_193, x_188, x_188); +lean_inc(x_1); +x_195 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1(x_19, x_1, x_21, x_22, x_23, x_194, x_6, x_7, x_185); +lean_dec(x_19); +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_12 = x_196; +x_13 = x_197; +goto block_18; +} +} +else +{ +lean_object* x_198; lean_object* x_199; lean_object* x_200; +lean_dec(x_23); +lean_dec(x_22); +lean_dec(x_21); +lean_dec(x_19); +x_198 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_198, 0, x_141); +x_199 = lean_box(0); +lean_inc(x_7); +lean_inc(x_6); +x_200 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__5(x_20, x_25, x_24, x_199, x_198, x_6, x_7, x_8); +lean_dec(x_20); +if (lean_obj_tag(x_200) == 0) +{ +lean_object* x_201; lean_object* x_202; +x_201 = lean_ctor_get(x_200, 0); +lean_inc(x_201); +x_202 = lean_ctor_get(x_200, 1); +lean_inc(x_202); +lean_dec(x_200); +x_12 = x_201; +x_13 = x_202; +goto block_18; +} +else +{ +uint8_t x_203; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_1); +x_203 = !lean_is_exclusive(x_200); +if (x_203 == 0) +{ +return x_200; +} +else +{ +lean_object* x_204; lean_object* x_205; lean_object* x_206; +x_204 = lean_ctor_get(x_200, 0); +x_205 = lean_ctor_get(x_200, 1); +lean_inc(x_205); +lean_inc(x_204); +lean_dec(x_200); +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_207; lean_object* x_208; lean_object* x_209; +lean_dec(x_83); +lean_dec(x_23); +lean_dec(x_22); +lean_dec(x_21); +lean_dec(x_19); +x_207 = lean_box(0); +x_208 = lean_box(0); +lean_inc(x_7); +lean_inc(x_6); +x_209 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__5(x_20, x_25, x_24, x_208, x_207, x_6, x_7, x_8); +lean_dec(x_20); +if (lean_obj_tag(x_209) == 0) +{ +lean_object* x_210; lean_object* x_211; +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_12 = x_210; +x_13 = x_211; +goto block_18; +} +else +{ +uint8_t x_212; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_1); +x_212 = !lean_is_exclusive(x_209); +if (x_212 == 0) +{ +return x_209; +} +else +{ +lean_object* x_213; lean_object* x_214; lean_object* x_215; +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_alloc_ctor(1, 2, 0); +lean_ctor_set(x_215, 0, x_213); +lean_ctor_set(x_215, 1, x_214); +return x_215; +} +} +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__2(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_3, x_2); +if (x_5 == 0) +{ +lean_dec(x_1); +return x_4; +} +else +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; size_t x_9; size_t x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_6 = lean_array_uget(x_4, x_3); +x_7 = lean_unsigned_to_nat(0u); +x_8 = lean_array_uset(x_4, x_3, x_7); +x_9 = 1; +x_10 = lean_usize_add(x_3, x_9); +x_11 = lean_ctor_get(x_6, 2); +lean_inc(x_11); +lean_dec(x_6); +lean_inc(x_1); +x_12 = l_Lean_Name_append(x_1, x_11); +x_13 = lean_array_uset(x_8, x_3, x_12); +x_3 = x_10; +x_4 = x_13; +goto _start; +} +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___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) { +_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_12; lean_object* x_13; lean_object* x_14; size_t x_15; size_t x_16; lean_object* x_17; +x_10 = lean_array_uget(x_1, x_3); +x_11 = lean_ctor_get(x_10, 4); +lean_inc(x_11); +x_12 = lean_ctor_get(x_10, 10); +lean_inc(x_12); +lean_dec(x_10); +x_13 = lean_ctor_get(x_4, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_4, 1); +lean_inc(x_14); +lean_dec(x_4); +x_15 = lean_array_size(x_12); +x_16 = 0; +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_11); +x_17 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1(x_11, x_12, x_15, x_16, x_13, x_5, x_6, x_7); +if (lean_obj_tag(x_17) == 0) +{ +lean_object* x_18; lean_object* x_19; size_t x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; size_t x_25; size_t x_26; +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); +lean_dec(x_17); +x_20 = lean_array_size(x_12); +lean_inc(x_11); +x_21 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__2(x_11, x_20, x_16, x_12); +x_22 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_22, 0, x_11); +lean_ctor_set(x_22, 1, x_21); +x_23 = lean_array_push(x_14, x_22); +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_18); +lean_ctor_set(x_24, 1, x_23); +x_25 = 1; +x_26 = lean_usize_add(x_3, x_25); +x_3 = x_26; +x_4 = x_24; +x_7 = x_19; +goto _start; +} +else +{ +uint8_t x_28; +lean_dec(x_14); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_6); +lean_dec(x_5); +x_28 = !lean_is_exclusive(x_17); +if (x_28 == 0) +{ +return x_17; +} +else +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_17, 0); +x_30 = lean_ctor_get(x_17, 1); +lean_inc(x_30); +lean_inc(x_29); +lean_dec(x_17); +x_31 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_31, 0, x_29); +lean_ctor_set(x_31, 1, x_30); +return x_31; +} +} +} +} +} +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__4(lean_object* x_1, size_t x_2, size_t x_3) { +_start: +{ +uint8_t x_4; +x_4 = lean_usize_dec_eq(x_2, x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; uint8_t x_7; +x_5 = lean_array_uget(x_1, x_2); +x_6 = lean_ctor_get(x_5, 10); +lean_inc(x_6); +lean_dec(x_5); +x_7 = l_Array_isEmpty___rarg(x_6); +lean_dec(x_6); +if (x_7 == 0) +{ +uint8_t x_8; +x_8 = 1; +return x_8; +} +else +{ +size_t x_9; size_t x_10; +x_9 = 1; +x_10 = lean_usize_add(x_2, x_9); +x_2 = x_10; +goto _start; +} +} +else +{ +uint8_t x_12; +x_12 = 0; +return x_12; +} +} +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("genMatcherCode", 14, 14); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__1___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_Inductive___hyg_8753____closed__1; +x_2 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__1___closed__1; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__1___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("elaboratingComputedFields", 25, 25); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__1___closed__3; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__1(lean_object* x_1) { +_start: +{ +uint8_t x_2; +x_2 = !lean_is_exclusive(x_1); +if (x_2 == 0) +{ +lean_object* x_3; lean_object* x_4; uint8_t x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; lean_object* x_9; +x_3 = lean_ctor_get(x_1, 1); +x_4 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__1___closed__2; +x_5 = 0; +x_6 = l_Lean_KVMap_setBool(x_3, x_4, x_5); +x_7 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__1___closed__4; +x_8 = 1; +x_9 = l_Lean_KVMap_setBool(x_6, x_7, x_8); +lean_ctor_set(x_1, 1, x_9); +return x_1; +} +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; uint8_t x_19; lean_object* x_20; uint8_t x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; lean_object* x_25; lean_object* x_26; +x_10 = lean_ctor_get(x_1, 0); +x_11 = lean_ctor_get(x_1, 1); +x_12 = lean_ctor_get(x_1, 2); +x_13 = lean_ctor_get(x_1, 3); +x_14 = lean_ctor_get(x_1, 4); +x_15 = lean_ctor_get(x_1, 5); +x_16 = lean_ctor_get(x_1, 6); +x_17 = lean_ctor_get(x_1, 7); +x_18 = lean_ctor_get(x_1, 8); +x_19 = lean_ctor_get_uint8(x_1, sizeof(void*)*9); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_dec(x_1); +x_20 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__1___closed__2; +x_21 = 0; +x_22 = l_Lean_KVMap_setBool(x_11, x_20, x_21); +x_23 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__1___closed__4; +x_24 = 1; +x_25 = l_Lean_KVMap_setBool(x_22, x_23, x_24); +x_26 = lean_alloc_ctor(0, 9, 1); +lean_ctor_set(x_26, 0, x_10); +lean_ctor_set(x_26, 1, x_25); +lean_ctor_set(x_26, 2, x_12); +lean_ctor_set(x_26, 3, x_13); +lean_ctor_set(x_26, 4, x_14); +lean_ctor_set(x_26, 5, x_15); +lean_ctor_set(x_26, 6, x_16); +lean_ctor_set(x_26, 7, x_17); +lean_ctor_set(x_26, 8, x_18); +lean_ctor_set_uint8(x_26, sizeof(void*)*9, x_19); +return x_26; +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +x_9 = l_Lean_Elab_ComputedFields_setComputedFields(x_1, x_4, x_5, x_6, x_7, x_8); +return x_9; +} +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__8___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_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mutual", 6, 6); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; +x_2 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__1; +x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__7; +x_4 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__2; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("end", 3, 3); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__1), 1, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3(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; lean_object* x_9; +x_6 = lean_array_size(x_1); +x_7 = 0; +x_8 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__1; +lean_inc(x_4); +lean_inc(x_3); +x_9 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__3(x_1, x_6, x_7, x_8, x_3, x_4, x_5); +if (lean_obj_tag(x_9) == 0) +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; +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, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_10, 1); +lean_inc(x_13); +lean_dec(x_10); +x_14 = l_Lean_Elab_Command_getRef(x_3, x_4, 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); +x_17 = 0; +x_18 = l_Lean_SourceInfo_fromRef(x_15, x_17); +lean_dec(x_15); +x_19 = l_Lean_Elab_Command_getCurrMacroScope(x_3, x_4, x_16); +x_20 = !lean_is_exclusive(x_19); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; +x_21 = lean_ctor_get(x_19, 1); +x_22 = lean_ctor_get(x_19, 0); +lean_dec(x_22); +x_23 = l_Lean_Elab_Command_getMainModule___rarg(x_4, x_21); +x_24 = !lean_is_exclusive(x_23); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; 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_23, 1); +x_26 = lean_ctor_get(x_23, 0); +lean_dec(x_26); +x_27 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__2; +lean_inc(x_18); +lean_ctor_set_tag(x_23, 2); +lean_ctor_set(x_23, 1, x_27); +lean_ctor_set(x_23, 0, x_18); +x_28 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; +x_29 = l_Array_append___rarg(x_28, x_12); +lean_dec(x_12); +x_30 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2; +lean_inc(x_18); +x_31 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_31, 0, x_18); +lean_ctor_set(x_31, 1, x_30); +lean_ctor_set(x_31, 2, x_29); +x_32 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__4; +lean_inc(x_18); +lean_ctor_set_tag(x_19, 2); +lean_ctor_set(x_19, 1, x_32); +lean_ctor_set(x_19, 0, x_18); +x_33 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__3; +x_34 = l_Lean_Syntax_node3(x_18, x_33, x_23, x_31, x_19); +x_35 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabCommand), 4, 1); +lean_closure_set(x_35, 0, x_34); +x_36 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__5; +lean_inc(x_4); +lean_inc(x_3); +x_37 = l_Lean_Elab_Command_withScope___rarg(x_36, x_35, x_3, x_4, x_25); +if (lean_obj_tag(x_37) == 0) +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; lean_object* x_42; +x_38 = lean_ctor_get(x_37, 1); +lean_inc(x_38); +lean_dec(x_37); +x_39 = lean_array_get_size(x_1); +x_40 = lean_unsigned_to_nat(0u); +x_41 = lean_nat_dec_lt(x_40, x_39); +lean_dec(x_39); +x_42 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__2___boxed), 8, 1); +lean_closure_set(x_42, 0, x_13); +if (x_41 == 0) +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_43 = l_Lean_Elab_Command_instInhabitedInductiveView; +x_44 = l_outOfBounds___rarg(x_43); +x_45 = lean_ctor_get(x_44, 4); +lean_inc(x_45); +lean_dec(x_44); +x_46 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withDeclName___rarg), 9, 2); +lean_closure_set(x_46, 0, x_45); +lean_closure_set(x_46, 1, x_42); +x_47 = l_Lean_Elab_Command_liftTermElabM___rarg(x_46, x_3, x_4, x_38); +lean_dec(x_4); +lean_dec(x_3); +return x_47; +} +else +{ +lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_48 = lean_array_fget(x_1, x_40); +x_49 = lean_ctor_get(x_48, 4); +lean_inc(x_49); +lean_dec(x_48); +x_50 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withDeclName___rarg), 9, 2); +lean_closure_set(x_50, 0, x_49); +lean_closure_set(x_50, 1, x_42); +x_51 = l_Lean_Elab_Command_liftTermElabM___rarg(x_50, x_3, x_4, x_38); +lean_dec(x_4); +lean_dec(x_3); +return x_51; +} +} +else +{ +uint8_t x_52; +lean_dec(x_13); +lean_dec(x_4); +lean_dec(x_3); +x_52 = !lean_is_exclusive(x_37); +if (x_52 == 0) +{ +return x_37; +} +else +{ +lean_object* x_53; lean_object* x_54; lean_object* x_55; +x_53 = lean_ctor_get(x_37, 0); +x_54 = lean_ctor_get(x_37, 1); +lean_inc(x_54); +lean_inc(x_53); +lean_dec(x_37); +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; 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_56 = lean_ctor_get(x_23, 1); +lean_inc(x_56); +lean_dec(x_23); +x_57 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__2; +lean_inc(x_18); +x_58 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_58, 0, x_18); +lean_ctor_set(x_58, 1, x_57); +x_59 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; +x_60 = l_Array_append___rarg(x_59, x_12); +lean_dec(x_12); +x_61 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2; +lean_inc(x_18); +x_62 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_62, 0, x_18); +lean_ctor_set(x_62, 1, x_61); +lean_ctor_set(x_62, 2, x_60); +x_63 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__4; +lean_inc(x_18); +lean_ctor_set_tag(x_19, 2); +lean_ctor_set(x_19, 1, x_63); +lean_ctor_set(x_19, 0, x_18); +x_64 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__3; +x_65 = l_Lean_Syntax_node3(x_18, x_64, x_58, x_62, x_19); +x_66 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabCommand), 4, 1); +lean_closure_set(x_66, 0, x_65); +x_67 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__5; +lean_inc(x_4); +lean_inc(x_3); +x_68 = l_Lean_Elab_Command_withScope___rarg(x_67, x_66, x_3, x_4, x_56); +if (lean_obj_tag(x_68) == 0) +{ +lean_object* x_69; lean_object* x_70; lean_object* x_71; uint8_t x_72; lean_object* x_73; +x_69 = lean_ctor_get(x_68, 1); +lean_inc(x_69); +lean_dec(x_68); +x_70 = lean_array_get_size(x_1); +x_71 = lean_unsigned_to_nat(0u); +x_72 = lean_nat_dec_lt(x_71, x_70); +lean_dec(x_70); +x_73 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__2___boxed), 8, 1); +lean_closure_set(x_73, 0, x_13); +if (x_72 == 0) +{ +lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; +x_74 = l_Lean_Elab_Command_instInhabitedInductiveView; +x_75 = l_outOfBounds___rarg(x_74); +x_76 = lean_ctor_get(x_75, 4); +lean_inc(x_76); +lean_dec(x_75); +x_77 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withDeclName___rarg), 9, 2); +lean_closure_set(x_77, 0, x_76); +lean_closure_set(x_77, 1, x_73); +x_78 = l_Lean_Elab_Command_liftTermElabM___rarg(x_77, x_3, x_4, x_69); +lean_dec(x_4); +lean_dec(x_3); +return x_78; +} +else +{ +lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; +x_79 = lean_array_fget(x_1, x_71); +x_80 = lean_ctor_get(x_79, 4); +lean_inc(x_80); +lean_dec(x_79); +x_81 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withDeclName___rarg), 9, 2); +lean_closure_set(x_81, 0, x_80); +lean_closure_set(x_81, 1, x_73); +x_82 = l_Lean_Elab_Command_liftTermElabM___rarg(x_81, x_3, x_4, x_69); +lean_dec(x_4); +lean_dec(x_3); +return x_82; +} +} +else +{ +lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; +lean_dec(x_13); +lean_dec(x_4); +lean_dec(x_3); +x_83 = lean_ctor_get(x_68, 0); +lean_inc(x_83); +x_84 = lean_ctor_get(x_68, 1); +lean_inc(x_84); +if (lean_is_exclusive(x_68)) { + lean_ctor_release(x_68, 0); + lean_ctor_release(x_68, 1); + x_85 = x_68; +} else { + lean_dec_ref(x_68); + x_85 = lean_box(0); +} +if (lean_is_scalar(x_85)) { + x_86 = lean_alloc_ctor(1, 2, 0); +} else { + x_86 = x_85; +} +lean_ctor_set(x_86, 0, x_83); +lean_ctor_set(x_86, 1, x_84); +return x_86; +} +} +} +else +{ +lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_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_87 = lean_ctor_get(x_19, 1); +lean_inc(x_87); +lean_dec(x_19); +x_88 = l_Lean_Elab_Command_getMainModule___rarg(x_4, x_87); +x_89 = lean_ctor_get(x_88, 1); +lean_inc(x_89); +if (lean_is_exclusive(x_88)) { + lean_ctor_release(x_88, 0); + lean_ctor_release(x_88, 1); + x_90 = x_88; +} else { + lean_dec_ref(x_88); + x_90 = lean_box(0); +} +x_91 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__2; +lean_inc(x_18); +if (lean_is_scalar(x_90)) { + x_92 = lean_alloc_ctor(2, 2, 0); +} else { + x_92 = x_90; + lean_ctor_set_tag(x_92, 2); +} +lean_ctor_set(x_92, 0, x_18); +lean_ctor_set(x_92, 1, x_91); +x_93 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; +x_94 = l_Array_append___rarg(x_93, x_12); +lean_dec(x_12); +x_95 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2; +lean_inc(x_18); +x_96 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_96, 0, x_18); +lean_ctor_set(x_96, 1, x_95); +lean_ctor_set(x_96, 2, x_94); +x_97 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__4; +lean_inc(x_18); +x_98 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_98, 0, x_18); +lean_ctor_set(x_98, 1, x_97); +x_99 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__3; +x_100 = l_Lean_Syntax_node3(x_18, x_99, x_92, x_96, x_98); +x_101 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabCommand), 4, 1); +lean_closure_set(x_101, 0, x_100); +x_102 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__5; +lean_inc(x_4); +lean_inc(x_3); +x_103 = l_Lean_Elab_Command_withScope___rarg(x_102, x_101, x_3, x_4, x_89); +if (lean_obj_tag(x_103) == 0) +{ +lean_object* x_104; lean_object* x_105; lean_object* x_106; uint8_t x_107; lean_object* x_108; +x_104 = lean_ctor_get(x_103, 1); +lean_inc(x_104); +lean_dec(x_103); +x_105 = lean_array_get_size(x_1); +x_106 = lean_unsigned_to_nat(0u); +x_107 = lean_nat_dec_lt(x_106, x_105); +lean_dec(x_105); +x_108 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__2___boxed), 8, 1); +lean_closure_set(x_108, 0, x_13); +if (x_107 == 0) +{ +lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; +x_109 = l_Lean_Elab_Command_instInhabitedInductiveView; +x_110 = l_outOfBounds___rarg(x_109); +x_111 = lean_ctor_get(x_110, 4); +lean_inc(x_111); +lean_dec(x_110); +x_112 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withDeclName___rarg), 9, 2); +lean_closure_set(x_112, 0, x_111); +lean_closure_set(x_112, 1, x_108); +x_113 = l_Lean_Elab_Command_liftTermElabM___rarg(x_112, x_3, x_4, x_104); +lean_dec(x_4); +lean_dec(x_3); +return x_113; +} +else +{ +lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; +x_114 = lean_array_fget(x_1, x_106); +x_115 = lean_ctor_get(x_114, 4); +lean_inc(x_115); +lean_dec(x_114); +x_116 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withDeclName___rarg), 9, 2); +lean_closure_set(x_116, 0, x_115); +lean_closure_set(x_116, 1, x_108); +x_117 = l_Lean_Elab_Command_liftTermElabM___rarg(x_116, x_3, x_4, x_104); +lean_dec(x_4); +lean_dec(x_3); +return x_117; +} +} +else +{ +lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; +lean_dec(x_13); +lean_dec(x_4); +lean_dec(x_3); +x_118 = lean_ctor_get(x_103, 0); +lean_inc(x_118); +x_119 = lean_ctor_get(x_103, 1); +lean_inc(x_119); +if (lean_is_exclusive(x_103)) { + lean_ctor_release(x_103, 0); + lean_ctor_release(x_103, 1); + x_120 = x_103; +} else { + lean_dec_ref(x_103); + x_120 = lean_box(0); +} +if (lean_is_scalar(x_120)) { + x_121 = lean_alloc_ctor(1, 2, 0); +} else { + x_121 = x_120; +} +lean_ctor_set(x_121, 0, x_118); +lean_ctor_set(x_121, 1, x_119); +return x_121; +} +} +} +else +{ +uint8_t x_122; +lean_dec(x_4); +lean_dec(x_3); +x_122 = !lean_is_exclusive(x_9); +if (x_122 == 0) +{ +return x_9; +} +else +{ +lean_object* x_123; lean_object* x_124; lean_object* x_125; +x_123 = lean_ctor_get(x_9, 0); +x_124 = lean_ctor_get(x_9, 1); +lean_inc(x_124); +lean_inc(x_123); +lean_dec(x_9); +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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields(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; +x_5 = lean_array_get_size(x_1); +x_6 = lean_unsigned_to_nat(0u); +x_7 = lean_nat_dec_lt(x_6, x_5); +if (x_7 == 0) +{ +lean_object* x_8; lean_object* x_9; +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +x_8 = lean_box(0); +x_9 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_9, 0, x_8); +lean_ctor_set(x_9, 1, x_4); +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_5); +lean_dec(x_5); +x_12 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__4(x_1, x_10, x_11); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_3); +lean_dec(x_2); +x_13 = lean_box(0); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_13); +lean_ctor_set(x_14, 1, x_4); +return x_14; +} +else +{ +lean_object* x_15; lean_object* x_16; +x_15 = lean_box(0); +x_16 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3(x_1, x_15, x_2, x_3, x_4); +return x_16; +} +} +} +} +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* x_1, lean_object* x_2, lean_object* x_3, 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_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_1); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___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: +{ +lean_object* x_11; +x_11 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___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_7); +lean_dec(x_1); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___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_6); +lean_dec(x_1); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_5); +lean_dec(x_1); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___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: +{ +lean_object* x_9; +x_9 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_4); +lean_dec(x_1); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +size_t x_9; size_t x_10; lean_object* x_11; +x_9 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_10 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_11 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1(x_1, x_2, x_9, x_10, x_5, x_6, x_7, x_8); +lean_dec(x_2); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___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; +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_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__2(x_1, x_5, x_6, x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___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) { +_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_dec(x_3); +x_10 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__3(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_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; size_t x_5; uint8_t x_6; lean_object* x_7; +x_4 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_5 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_6 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__4(x_1, x_4, x_5); +lean_dec(x_1); +x_7 = lean_box(x_6); +return x_7; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +x_9 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_3); +lean_dec(x_2); +return x_9; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_2); +lean_dec(x_1); +return x_6; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___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_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields(x_1, x_2, x_3, x_4); +lean_dec(x_1); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInductiveViews___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); +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_dec(x_4); +x_14 = lean_array_uget(x_1, x_3); +x_15 = lean_ctor_get(x_14, 4); +lean_inc(x_15); +lean_dec(x_14); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +x_16 = l_Lean_Meta_mkInjectiveTheorems(x_15, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_16) == 0) +{ +lean_object* x_17; size_t x_18; size_t x_19; lean_object* x_20; +x_17 = lean_ctor_get(x_16, 1); +lean_inc(x_17); +lean_dec(x_16); +x_18 = 1; +x_19 = lean_usize_add(x_3, x_18); +x_20 = lean_box(0); +x_3 = x_19; +x_4 = x_20; +x_11 = x_17; +goto _start; +} +else +{ +uint8_t x_22; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +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; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInductiveViews___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; +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); +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); +x_15 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl(x_2, x_3, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_15) == 0) +{ +lean_object* x_16; lean_object* x_17; +x_16 = lean_ctor_get(x_15, 1); +lean_inc(x_16); +lean_dec(x_15); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_4); +x_17 = l_Lean_Meta_mkSizeOfInstances(x_4, x_7, x_8, x_9, x_10, x_16); +if (lean_obj_tag(x_17) == 0) +{ +lean_object* x_18; lean_object* x_19; +x_18 = lean_ctor_get(x_17, 1); +lean_inc(x_18); +lean_dec(x_17); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +x_19 = l_Lean_Meta_IndPredBelow_mkBelow(x_4, x_7, x_8, x_9, x_10, x_18); +if (lean_obj_tag(x_19) == 0) +{ +lean_object* x_20; size_t x_21; size_t x_22; lean_object* x_23; lean_object* x_24; +x_20 = lean_ctor_get(x_19, 1); +lean_inc(x_20); +lean_dec(x_19); +x_21 = lean_array_size(x_3); +x_22 = 0; +x_23 = lean_box(0); +x_24 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInductiveViews___spec__1(x_3, x_21, x_22, x_23, x_5, x_6, x_7, x_8, x_9, x_10, x_20); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +if (lean_obj_tag(x_24) == 0) +{ +uint8_t x_25; +x_25 = !lean_is_exclusive(x_24); +if (x_25 == 0) +{ +lean_object* x_26; +x_26 = lean_ctor_get(x_24, 0); +lean_dec(x_26); +lean_ctor_set(x_24, 0, x_23); +return x_24; +} +else +{ +lean_object* x_27; lean_object* x_28; +x_27 = lean_ctor_get(x_24, 1); +lean_inc(x_27); +lean_dec(x_24); +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_23); +lean_ctor_set(x_28, 1, x_27); +return x_28; +} +} +else +{ +uint8_t x_29; +x_29 = !lean_is_exclusive(x_24); +if (x_29 == 0) +{ +return x_24; +} +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; +} +} +} +else +{ +uint8_t x_33; +lean_dec(x_9); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +x_33 = !lean_is_exclusive(x_19); +if (x_33 == 0) +{ +return x_19; +} +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_19, 0); +x_35 = lean_ctor_get(x_19, 1); +lean_inc(x_35); +lean_inc(x_34); +lean_dec(x_19); +x_36 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_36, 0, x_34); +lean_ctor_set(x_36, 1, x_35); +return x_36; +} +} +} +else +{ +uint8_t x_37; +lean_dec(x_9); +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); +x_37 = !lean_is_exclusive(x_17); +if (x_37 == 0) +{ +return x_17; +} +else +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_17, 0); +x_39 = lean_ctor_get(x_17, 1); +lean_inc(x_39); +lean_inc(x_38); +lean_dec(x_17); +x_40 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +return x_40; +} +} +} +else +{ +uint8_t x_41; +lean_dec(x_9); +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); +x_41 = !lean_is_exclusive(x_15); +if (x_41 == 0) +{ +return x_15; +} +else +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_42 = lean_ctor_get(x_15, 0); +x_43 = lean_ctor_get(x_15, 1); +lean_inc(x_43); +lean_inc(x_42); +lean_dec(x_15); +x_44 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_44, 0, x_42); +lean_ctor_set(x_44, 1, x_43); +return x_44; +} +} +} +else +{ +lean_object* x_45; lean_object* x_46; 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; lean_object* x_57; uint8_t x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; +x_45 = lean_ctor_get(x_9, 0); +x_46 = lean_ctor_get(x_9, 1); +x_47 = lean_ctor_get(x_9, 2); +x_48 = lean_ctor_get(x_9, 3); +x_49 = lean_ctor_get(x_9, 4); +x_50 = lean_ctor_get(x_9, 5); +x_51 = lean_ctor_get(x_9, 6); +x_52 = lean_ctor_get(x_9, 7); +x_53 = lean_ctor_get(x_9, 8); +x_54 = lean_ctor_get(x_9, 9); +x_55 = lean_ctor_get(x_9, 10); +x_56 = lean_ctor_get_uint8(x_9, sizeof(void*)*12); +x_57 = lean_ctor_get(x_9, 11); +x_58 = lean_ctor_get_uint8(x_9, sizeof(void*)*12 + 1); +lean_inc(x_57); +lean_inc(x_55); +lean_inc(x_54); +lean_inc(x_53); +lean_inc(x_52); +lean_inc(x_51); +lean_inc(x_50); +lean_inc(x_49); +lean_inc(x_48); +lean_inc(x_47); +lean_inc(x_46); +lean_inc(x_45); +lean_dec(x_9); +x_59 = l_Lean_replaceRef(x_1, x_50); +lean_dec(x_50); +x_60 = lean_alloc_ctor(0, 12, 2); +lean_ctor_set(x_60, 0, x_45); +lean_ctor_set(x_60, 1, x_46); +lean_ctor_set(x_60, 2, x_47); +lean_ctor_set(x_60, 3, x_48); +lean_ctor_set(x_60, 4, x_49); +lean_ctor_set(x_60, 5, x_59); +lean_ctor_set(x_60, 6, x_51); +lean_ctor_set(x_60, 7, x_52); +lean_ctor_set(x_60, 8, x_53); +lean_ctor_set(x_60, 9, x_54); +lean_ctor_set(x_60, 10, x_55); +lean_ctor_set(x_60, 11, x_57); +lean_ctor_set_uint8(x_60, sizeof(void*)*12, x_56); +lean_ctor_set_uint8(x_60, sizeof(void*)*12 + 1, x_58); +lean_inc(x_10); +lean_inc(x_60); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_3); +x_61 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl(x_2, x_3, x_5, x_6, x_7, x_8, x_60, x_10, x_11); +if (lean_obj_tag(x_61) == 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); +lean_inc(x_10); +lean_inc(x_60); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_4); +x_63 = l_Lean_Meta_mkSizeOfInstances(x_4, x_7, x_8, x_60, x_10, x_62); +if (lean_obj_tag(x_63) == 0) +{ +lean_object* x_64; lean_object* x_65; +x_64 = lean_ctor_get(x_63, 1); +lean_inc(x_64); +lean_dec(x_63); +lean_inc(x_10); +lean_inc(x_60); +lean_inc(x_8); +lean_inc(x_7); +x_65 = l_Lean_Meta_IndPredBelow_mkBelow(x_4, x_7, x_8, x_60, x_10, x_64); +if (lean_obj_tag(x_65) == 0) +{ +lean_object* x_66; size_t x_67; size_t x_68; lean_object* x_69; lean_object* x_70; +x_66 = lean_ctor_get(x_65, 1); +lean_inc(x_66); +lean_dec(x_65); +x_67 = lean_array_size(x_3); +x_68 = 0; +x_69 = lean_box(0); +x_70 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInductiveViews___spec__1(x_3, x_67, x_68, x_69, x_5, x_6, x_7, x_8, x_60, x_10, x_66); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +if (lean_obj_tag(x_70) == 0) +{ +lean_object* x_71; lean_object* x_72; lean_object* x_73; +x_71 = lean_ctor_get(x_70, 1); +lean_inc(x_71); +if (lean_is_exclusive(x_70)) { + lean_ctor_release(x_70, 0); + lean_ctor_release(x_70, 1); + x_72 = x_70; +} else { + lean_dec_ref(x_70); + x_72 = lean_box(0); +} +if (lean_is_scalar(x_72)) { + x_73 = lean_alloc_ctor(0, 2, 0); +} else { + x_73 = x_72; +} +lean_ctor_set(x_73, 0, x_69); +lean_ctor_set(x_73, 1, x_71); +return x_73; +} +else +{ +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); +x_75 = lean_ctor_get(x_70, 1); +lean_inc(x_75); +if (lean_is_exclusive(x_70)) { + lean_ctor_release(x_70, 0); + lean_ctor_release(x_70, 1); + x_76 = x_70; +} else { + lean_dec_ref(x_70); + x_76 = lean_box(0); +} +if (lean_is_scalar(x_76)) { + x_77 = lean_alloc_ctor(1, 2, 0); +} else { + x_77 = x_76; +} +lean_ctor_set(x_77, 0, x_74); +lean_ctor_set(x_77, 1, x_75); +return x_77; +} +} +else +{ +lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +lean_dec(x_60); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +x_78 = lean_ctor_get(x_65, 0); +lean_inc(x_78); +x_79 = lean_ctor_get(x_65, 1); +lean_inc(x_79); +if (lean_is_exclusive(x_65)) { + lean_ctor_release(x_65, 0); + lean_ctor_release(x_65, 1); + x_80 = x_65; +} else { + lean_dec_ref(x_65); + x_80 = lean_box(0); +} +if (lean_is_scalar(x_80)) { + x_81 = lean_alloc_ctor(1, 2, 0); +} else { + x_81 = x_80; +} +lean_ctor_set(x_81, 0, x_78); +lean_ctor_set(x_81, 1, x_79); +return x_81; +} +} +else +{ +lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; +lean_dec(x_60); +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); +x_82 = lean_ctor_get(x_63, 0); +lean_inc(x_82); +x_83 = lean_ctor_get(x_63, 1); +lean_inc(x_83); +if (lean_is_exclusive(x_63)) { + lean_ctor_release(x_63, 0); + lean_ctor_release(x_63, 1); + x_84 = x_63; +} else { + lean_dec_ref(x_63); + x_84 = lean_box(0); +} +if (lean_is_scalar(x_84)) { + x_85 = lean_alloc_ctor(1, 2, 0); +} else { + x_85 = x_84; +} +lean_ctor_set(x_85, 0, x_82); +lean_ctor_set(x_85, 1, x_83); +return x_85; +} +} +else +{ +lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; +lean_dec(x_60); +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); +x_86 = lean_ctor_get(x_61, 0); +lean_inc(x_86); +x_87 = lean_ctor_get(x_61, 1); +lean_inc(x_87); +if (lean_is_exclusive(x_61)) { + lean_ctor_release(x_61, 0); + lean_ctor_release(x_61, 1); + x_88 = x_61; +} else { + lean_dec_ref(x_61); + x_88 = lean_box(0); +} +if (lean_is_scalar(x_88)) { + x_89 = lean_alloc_ctor(1, 2, 0); +} else { + x_89 = x_88; +} +lean_ctor_set(x_89, 0, x_86); +lean_ctor_set(x_89, 1, x_87); +return x_89; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInductiveViews(lean_object* x_1, lean_object* x_2, lean_object* x_3, 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_16; lean_object* x_17; uint8_t x_18; +x_16 = lean_array_get_size(x_2); +x_17 = lean_unsigned_to_nat(0u); +x_18 = lean_nat_dec_lt(x_17, x_16); +lean_dec(x_16); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; +x_19 = l_Lean_Elab_Command_instInhabitedInductiveView; +x_20 = l_outOfBounds___rarg(x_19); +x_10 = x_20; +goto block_15; +} +else +{ +lean_object* x_21; +x_21 = lean_array_fget(x_2, x_17); +x_10 = x_21; +goto block_15; +} +block_15: +{ +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, 4); +lean_inc(x_12); +lean_dec(x_10); +lean_inc(x_12); +x_13 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabInductiveViews___lambda__1___boxed), 11, 4); +lean_closure_set(x_13, 0, x_11); +lean_closure_set(x_13, 1, x_1); +lean_closure_set(x_13, 2, x_2); +lean_closure_set(x_13, 3, x_12); +x_14 = l_Lean_Elab_Term_withDeclName___rarg(x_12, x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_14; +} +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInductiveViews___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_Command_elabInductiveViews___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; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInductiveViews___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, 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_Command_elabInductiveViews___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_1); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInductiveViewsPostprocessing___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_17; uint8_t x_18; lean_object* x_19; +lean_dec(x_4); +x_14 = lean_array_uget(x_1, x_3); +x_15 = lean_ctor_get(x_14, 4); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 2); +lean_inc(x_16); +lean_dec(x_14); +x_17 = lean_ctor_get(x_16, 2); +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); +if (lean_obj_tag(x_19) == 0) +{ +lean_object* x_20; size_t x_21; size_t x_22; lean_object* x_23; +x_20 = lean_ctor_get(x_19, 1); +lean_inc(x_20); +lean_dec(x_19); +x_21 = 1; +x_22 = lean_usize_add(x_3, x_21); +x_23 = lean_box(0); +x_3 = x_22; +x_4 = x_23; +x_11 = x_20; +goto _start; +} +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) +{ +return x_19; +} +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_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_EXPORT lean_object* l_Lean_Elab_Command_elabInductiveViewsPostprocessing___lambda__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) { +_start: +{ +uint8_t x_12; +x_12 = !lean_is_exclusive(x_9); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +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 = lean_box(0); +x_16 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInductiveViewsPostprocessing___spec__1(x_2, x_3, x_4, x_15, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_16) == 0) +{ +uint8_t x_17; +x_17 = !lean_is_exclusive(x_16); +if (x_17 == 0) +{ +lean_object* x_18; +x_18 = lean_ctor_get(x_16, 0); +lean_dec(x_18); +lean_ctor_set(x_16, 0, x_15); +return x_16; +} +else +{ +lean_object* x_19; lean_object* x_20; +x_19 = lean_ctor_get(x_16, 1); +lean_inc(x_19); +lean_dec(x_16); +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_15); +lean_ctor_set(x_20, 1, x_19); +return x_20; +} +} +else +{ +uint8_t x_21; +x_21 = !lean_is_exclusive(x_16); +if (x_21 == 0) +{ +return x_16; +} +else +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_16, 0); +x_23 = lean_ctor_get(x_16, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_16); +x_24 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); +return x_24; +} +} +} +else +{ +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; uint8_t x_36; lean_object* x_37; uint8_t x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_25 = lean_ctor_get(x_9, 0); +x_26 = lean_ctor_get(x_9, 1); +x_27 = lean_ctor_get(x_9, 2); +x_28 = lean_ctor_get(x_9, 3); +x_29 = lean_ctor_get(x_9, 4); +x_30 = lean_ctor_get(x_9, 5); +x_31 = lean_ctor_get(x_9, 6); +x_32 = lean_ctor_get(x_9, 7); +x_33 = lean_ctor_get(x_9, 8); +x_34 = lean_ctor_get(x_9, 9); +x_35 = lean_ctor_get(x_9, 10); +x_36 = lean_ctor_get_uint8(x_9, sizeof(void*)*12); +x_37 = lean_ctor_get(x_9, 11); +x_38 = lean_ctor_get_uint8(x_9, sizeof(void*)*12 + 1); +lean_inc(x_37); +lean_inc(x_35); +lean_inc(x_34); +lean_inc(x_33); +lean_inc(x_32); +lean_inc(x_31); +lean_inc(x_30); +lean_inc(x_29); +lean_inc(x_28); +lean_inc(x_27); +lean_inc(x_26); +lean_inc(x_25); +lean_dec(x_9); +x_39 = l_Lean_replaceRef(x_1, x_30); +lean_dec(x_30); +x_40 = lean_alloc_ctor(0, 12, 2); +lean_ctor_set(x_40, 0, x_25); +lean_ctor_set(x_40, 1, x_26); +lean_ctor_set(x_40, 2, x_27); +lean_ctor_set(x_40, 3, x_28); +lean_ctor_set(x_40, 4, x_29); +lean_ctor_set(x_40, 5, x_39); +lean_ctor_set(x_40, 6, x_31); +lean_ctor_set(x_40, 7, x_32); +lean_ctor_set(x_40, 8, x_33); +lean_ctor_set(x_40, 9, x_34); +lean_ctor_set(x_40, 10, x_35); +lean_ctor_set(x_40, 11, x_37); +lean_ctor_set_uint8(x_40, sizeof(void*)*12, x_36); +lean_ctor_set_uint8(x_40, sizeof(void*)*12 + 1, x_38); +x_41 = lean_box(0); +x_42 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInductiveViewsPostprocessing___spec__1(x_2, x_3, x_4, x_41, x_5, x_6, x_7, x_8, x_40, x_10, x_11); +if (lean_obj_tag(x_42) == 0) +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; +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_42); + x_44 = lean_box(0); +} +if (lean_is_scalar(x_44)) { + x_45 = lean_alloc_ctor(0, 2, 0); +} else { + x_45 = x_44; +} +lean_ctor_set(x_45, 0, x_41); +lean_ctor_set(x_45, 1, x_43); +return x_45; +} +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); +lean_inc(x_46); +x_47 = lean_ctor_get(x_42, 1); +lean_inc(x_47); +if (lean_is_exclusive(x_42)) { + lean_ctor_release(x_42, 0); + lean_ctor_release(x_42, 1); + x_48 = x_42; +} else { + lean_dec_ref(x_42); + x_48 = lean_box(0); +} +if (lean_is_scalar(x_48)) { + x_49 = lean_alloc_ctor(1, 2, 0); +} else { + x_49 = x_48; +} +lean_ctor_set(x_49, 0, x_46); +lean_ctor_set(x_49, 1, x_47); +return x_49; +} +} +} +} +static lean_object* _init_l_Lean_Elab_Command_elabInductiveViewsPostprocessing___lambda__2___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_Elab_Command_elabInductiveViewsPostprocessing___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; size_t 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, 4); +lean_inc(x_12); +lean_dec(x_1); +x_13 = lean_array_size(x_2); +x_14 = lean_box_usize(x_13); +x_15 = l_Lean_Elab_Command_elabInductiveViewsPostprocessing___lambda__2___boxed__const__1; +x_16 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabInductiveViewsPostprocessing___lambda__1___boxed), 11, 4); +lean_closure_set(x_16, 0, x_3); +lean_closure_set(x_16, 1, x_2); +lean_closure_set(x_16, 2, x_14); +lean_closure_set(x_16, 3, x_15); +x_17 = l_Lean_Elab_Term_withDeclName___rarg(x_12, x_16, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_17; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInductiveViewsPostprocessing(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_object* x_8; lean_object* x_9; +x_5 = lean_array_get_size(x_1); +x_6 = lean_unsigned_to_nat(0u); +x_7 = lean_nat_dec_lt(x_6, x_5); +lean_dec(x_5); +lean_inc(x_3); +lean_inc(x_2); +x_8 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields(x_1, x_2, x_3, x_4); +if (x_7 == 0) +{ +lean_object* x_25; lean_object* x_26; +x_25 = l_Lean_Elab_Command_instInhabitedInductiveView; +x_26 = l_outOfBounds___rarg(x_25); +x_9 = x_26; +goto block_24; +} +else +{ +lean_object* x_27; +x_27 = lean_array_fget(x_1, x_6); +x_9 = x_27; +goto block_24; +} +block_24: +{ +if (lean_obj_tag(x_8) == 0) +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_8, 1); +lean_inc(x_10); +lean_dec(x_8); +x_11 = lean_ctor_get(x_9, 0); +lean_inc(x_11); +lean_inc(x_3); +lean_inc(x_2); +x_12 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers(x_1, x_2, x_3, x_10); +if (lean_obj_tag(x_12) == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_12, 1); +lean_inc(x_13); +lean_dec(x_12); +x_14 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabInductiveViewsPostprocessing___lambda__2___boxed), 11, 3); +lean_closure_set(x_14, 0, x_9); +lean_closure_set(x_14, 1, x_1); +lean_closure_set(x_14, 2, x_11); +x_15 = l_Lean_Elab_Command_runTermElabM___rarg(x_14, x_2, x_3, x_13); +lean_dec(x_3); +lean_dec(x_2); +return x_15; +} +else +{ +uint8_t x_16; +lean_dec(x_11); +lean_dec(x_9); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_16 = !lean_is_exclusive(x_12); +if (x_16 == 0) +{ +return x_12; +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_12, 0); +x_18 = lean_ctor_get(x_12, 1); +lean_inc(x_18); +lean_inc(x_17); +lean_dec(x_12); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set(x_19, 1, x_18); +return x_19; +} +} } 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_54, 1); -lean_inc(x_69); -lean_dec(x_54); -x_70 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__12; -x_71 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; -lean_inc(x_51); -x_72 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_72, 0, x_51); -lean_ctor_set(x_72, 1, x_70); -lean_ctor_set(x_72, 2, x_71); -x_73 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; -lean_inc(x_51); -x_74 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_74, 0, x_51); -lean_ctor_set(x_74, 1, x_73); -x_75 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; -lean_inc(x_51); -x_76 = l_Lean_Syntax_node1(x_51, x_75, x_74); -lean_inc(x_51); -x_77 = l_Lean_Syntax_node1(x_51, x_70, x_76); -lean_inc_n(x_72, 4); -x_78 = l_Lean_Syntax_node6(x_51, x_25, x_72, x_72, x_72, x_77, x_72, x_72); -lean_inc(x_1); -x_79 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1(x_19, x_1, x_21, x_22, x_23, x_78, x_6, x_7, x_69); -lean_dec(x_19); -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_12 = x_80; -x_13 = x_81; -goto block_18; -} +uint8_t x_20; +lean_dec(x_9); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_20 = !lean_is_exclusive(x_8); +if (x_20 == 0) +{ +return x_8; } else { -lean_object* x_82; lean_object* x_83; uint8_t x_84; -x_82 = lean_unsigned_to_nat(0u); -x_83 = l_Lean_Syntax_getArg(x_20, x_82); -x_84 = l_Lean_Syntax_isNone(x_83); -if (x_84 == 0) +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_8, 0); +x_22 = lean_ctor_get(x_8, 1); +lean_inc(x_22); +lean_inc(x_21); +lean_dec(x_8); +x_23 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_23, 0, x_21); +lean_ctor_set(x_23, 1, x_22); +return x_23; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInductiveViewsPostprocessing___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_85; uint8_t x_86; -x_85 = lean_unsigned_to_nat(1u); -lean_inc(x_83); -x_86 = l_Lean_Syntax_matchesNull(x_83, x_85); -if (x_86 == 0) +size_t x_12; size_t x_13; lean_object* x_14; +x_12 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_13 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_14 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInductiveViewsPostprocessing___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; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInductiveViewsPostprocessing___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, 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_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; uint8_t 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; uint8_t x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; uint8_t x_114; -lean_dec(x_83); -lean_dec(x_24); -x_87 = l_Lean_Elab_Command_getRef(x_6, x_7, x_8); -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); -x_90 = l_Lean_replaceRef(x_20, x_88); -lean_dec(x_88); -lean_dec(x_20); -x_91 = lean_ctor_get(x_6, 0); -lean_inc(x_91); -x_92 = lean_ctor_get(x_6, 1); -lean_inc(x_92); -x_93 = lean_ctor_get(x_6, 2); -lean_inc(x_93); -x_94 = lean_ctor_get(x_6, 3); -lean_inc(x_94); -x_95 = lean_ctor_get(x_6, 4); -lean_inc(x_95); -x_96 = lean_ctor_get(x_6, 5); -lean_inc(x_96); -x_97 = lean_ctor_get(x_6, 7); -lean_inc(x_97); -x_98 = lean_ctor_get(x_6, 8); -lean_inc(x_98); -x_99 = lean_ctor_get(x_6, 9); -lean_inc(x_99); -x_100 = lean_ctor_get_uint8(x_6, sizeof(void*)*10); -x_101 = lean_alloc_ctor(0, 10, 1); -lean_ctor_set(x_101, 0, x_91); -lean_ctor_set(x_101, 1, x_92); -lean_ctor_set(x_101, 2, x_93); -lean_ctor_set(x_101, 3, x_94); -lean_ctor_set(x_101, 4, x_95); -lean_ctor_set(x_101, 5, x_96); -lean_ctor_set(x_101, 6, x_90); -lean_ctor_set(x_101, 7, x_97); -lean_ctor_set(x_101, 8, x_98); -lean_ctor_set(x_101, 9, x_99); -lean_ctor_set_uint8(x_101, sizeof(void*)*10, x_100); -x_102 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__3; -x_103 = 2; -x_104 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_102, x_103, x_101, x_7, x_89); -x_105 = lean_ctor_get(x_104, 1); -lean_inc(x_105); -lean_dec(x_104); -x_106 = l_Lean_Elab_Command_getRef(x_6, x_7, 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 = 0; -x_110 = l_Lean_SourceInfo_fromRef(x_107, x_109); -lean_dec(x_107); -x_111 = l_Lean_Elab_Command_getCurrMacroScope(x_6, x_7, x_108); -x_112 = lean_ctor_get(x_111, 1); -lean_inc(x_112); -lean_dec(x_111); -x_113 = l_Lean_Elab_Command_getMainModule___rarg(x_7, x_112); -x_114 = !lean_is_exclusive(x_113); -if (x_114 == 0) +size_t x_12; size_t x_13; lean_object* x_14; +x_12 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_13 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_14 = l_Lean_Elab_Command_elabInductiveViewsPostprocessing___lambda__1(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_2); +lean_dec(x_1); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInductiveViewsPostprocessing___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: { -lean_object* x_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_115 = lean_ctor_get(x_113, 1); -x_116 = lean_ctor_get(x_113, 0); -lean_dec(x_116); -x_117 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__12; -x_118 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; -lean_inc(x_110); -x_119 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_119, 0, x_110); -lean_ctor_set(x_119, 1, x_117); -lean_ctor_set(x_119, 2, x_118); -x_120 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; -lean_inc(x_110); -lean_ctor_set_tag(x_113, 2); -lean_ctor_set(x_113, 1, x_120); -lean_ctor_set(x_113, 0, x_110); -x_121 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; -lean_inc(x_110); -x_122 = l_Lean_Syntax_node1(x_110, x_121, x_113); -lean_inc(x_110); -x_123 = l_Lean_Syntax_node1(x_110, x_117, x_122); -lean_inc_n(x_119, 4); -x_124 = l_Lean_Syntax_node6(x_110, x_25, x_119, x_119, x_119, x_123, x_119, x_119); -lean_inc(x_1); -x_125 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1(x_19, x_1, x_21, x_22, x_23, x_124, x_6, x_7, x_115); -lean_dec(x_19); -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_12 = x_126; -x_13 = x_127; -goto block_18; +lean_object* x_12; +x_12 = l_Lean_Elab_Command_elabInductiveViewsPostprocessing___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_4); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabInductives___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_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +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_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; -x_128 = lean_ctor_get(x_113, 1); -lean_inc(x_128); -lean_dec(x_113); -x_129 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__12; -x_130 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; -lean_inc(x_110); -x_131 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_131, 0, x_110); -lean_ctor_set(x_131, 1, x_129); -lean_ctor_set(x_131, 2, x_130); -x_132 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; -lean_inc(x_110); -x_133 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_133, 0, x_110); -lean_ctor_set(x_133, 1, x_132); -x_134 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; -lean_inc(x_110); -x_135 = l_Lean_Syntax_node1(x_110, x_134, x_133); -lean_inc(x_110); -x_136 = l_Lean_Syntax_node1(x_110, x_129, x_135); -lean_inc_n(x_131, 4); -x_137 = l_Lean_Syntax_node6(x_110, x_25, x_131, x_131, x_131, x_136, x_131, x_131); -lean_inc(x_1); -x_138 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1(x_19, x_1, x_21, x_22, x_23, x_137, x_6, x_7, x_128); -lean_dec(x_19); -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_12 = x_139; -x_13 = x_140; -goto block_18; +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_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, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_13, 1); +lean_inc(x_17); +lean_dec(x_13); +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_18 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView(x_16, 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; 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); +lean_dec(x_5); +lean_dec(x_4); +x_25 = !lean_is_exclusive(x_18); +if (x_25 == 0) +{ +return x_18; } else { -lean_object* x_141; lean_object* x_142; uint8_t x_143; -x_141 = l_Lean_Syntax_getArg(x_83, x_82); -lean_dec(x_83); -x_142 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___closed__4; -lean_inc(x_141); -x_143 = l_Lean_Syntax_isOfKind(x_141, x_142); -if (x_143 == 0) +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_Command_elabInductives___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_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; uint8_t x_157; lean_object* x_158; lean_object* x_159; uint8_t x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; uint8_t x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; uint8_t x_171; -lean_dec(x_141); -lean_dec(x_24); -x_144 = l_Lean_Elab_Command_getRef(x_6, x_7, x_8); -x_145 = lean_ctor_get(x_144, 0); -lean_inc(x_145); -x_146 = lean_ctor_get(x_144, 1); -lean_inc(x_146); -lean_dec(x_144); -x_147 = l_Lean_replaceRef(x_20, x_145); -lean_dec(x_145); -lean_dec(x_20); -x_148 = lean_ctor_get(x_6, 0); -lean_inc(x_148); -x_149 = lean_ctor_get(x_6, 1); -lean_inc(x_149); -x_150 = lean_ctor_get(x_6, 2); -lean_inc(x_150); -x_151 = lean_ctor_get(x_6, 3); -lean_inc(x_151); -x_152 = lean_ctor_get(x_6, 4); -lean_inc(x_152); -x_153 = lean_ctor_get(x_6, 5); -lean_inc(x_153); -x_154 = lean_ctor_get(x_6, 7); -lean_inc(x_154); -x_155 = lean_ctor_get(x_6, 8); -lean_inc(x_155); -x_156 = lean_ctor_get(x_6, 9); -lean_inc(x_156); -x_157 = lean_ctor_get_uint8(x_6, sizeof(void*)*10); -x_158 = lean_alloc_ctor(0, 10, 1); -lean_ctor_set(x_158, 0, x_148); -lean_ctor_set(x_158, 1, x_149); -lean_ctor_set(x_158, 2, x_150); -lean_ctor_set(x_158, 3, x_151); -lean_ctor_set(x_158, 4, x_152); -lean_ctor_set(x_158, 5, x_153); -lean_ctor_set(x_158, 6, x_147); -lean_ctor_set(x_158, 7, x_154); -lean_ctor_set(x_158, 8, x_155); -lean_ctor_set(x_158, 9, x_156); -lean_ctor_set_uint8(x_158, sizeof(void*)*10, x_157); -x_159 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__3; -x_160 = 2; -x_161 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_159, x_160, x_158, x_7, x_146); -x_162 = lean_ctor_get(x_161, 1); -lean_inc(x_162); -lean_dec(x_161); -x_163 = l_Lean_Elab_Command_getRef(x_6, x_7, x_162); -x_164 = lean_ctor_get(x_163, 0); -lean_inc(x_164); -x_165 = lean_ctor_get(x_163, 1); -lean_inc(x_165); -lean_dec(x_163); -x_166 = 0; -x_167 = l_Lean_SourceInfo_fromRef(x_164, x_166); -lean_dec(x_164); -x_168 = l_Lean_Elab_Command_getCurrMacroScope(x_6, x_7, x_165); -x_169 = lean_ctor_get(x_168, 1); -lean_inc(x_169); -lean_dec(x_168); -x_170 = l_Lean_Elab_Command_getMainModule___rarg(x_7, x_169); -x_171 = !lean_is_exclusive(x_170); -if (x_171 == 0) +size_t x_10; size_t x_11; lean_object* x_12; +x_10 = lean_array_size(x_1); +x_11 = 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_12 = l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabInductives___spec__1(x_10, x_11, x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_12) == 0) { -lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; -x_172 = lean_ctor_get(x_170, 1); -x_173 = lean_ctor_get(x_170, 0); -lean_dec(x_173); -x_174 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__12; -x_175 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; -lean_inc(x_167); -x_176 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_176, 0, x_167); -lean_ctor_set(x_176, 1, x_174); -lean_ctor_set(x_176, 2, x_175); -x_177 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; -lean_inc(x_167); -lean_ctor_set_tag(x_170, 2); -lean_ctor_set(x_170, 1, x_177); -lean_ctor_set(x_170, 0, x_167); -x_178 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; -lean_inc(x_167); -x_179 = l_Lean_Syntax_node1(x_167, x_178, x_170); -lean_inc(x_167); -x_180 = l_Lean_Syntax_node1(x_167, x_174, x_179); -lean_inc_n(x_176, 4); -x_181 = l_Lean_Syntax_node6(x_167, x_25, x_176, x_176, x_176, x_180, x_176, x_176); -lean_inc(x_1); -x_182 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1(x_19, x_1, x_21, x_22, x_23, x_181, x_6, x_7, x_172); -lean_dec(x_19); -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_12 = x_183; -x_13 = x_184; -goto block_18; +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_12, 1); +lean_inc(x_14); +lean_dec(x_12); +lean_inc(x_13); +x_15 = l_Lean_Elab_Command_elabInductiveViews(x_2, x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_14); +if (lean_obj_tag(x_15) == 0) +{ +uint8_t x_16; +x_16 = !lean_is_exclusive(x_15); +if (x_16 == 0) +{ +lean_object* x_17; +x_17 = lean_ctor_get(x_15, 0); +lean_dec(x_17); +lean_ctor_set(x_15, 0, x_13); +return x_15; } else { -lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; 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_185 = lean_ctor_get(x_170, 1); -lean_inc(x_185); -lean_dec(x_170); -x_186 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__12; -x_187 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; -lean_inc(x_167); -x_188 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_188, 0, x_167); -lean_ctor_set(x_188, 1, x_186); -lean_ctor_set(x_188, 2, x_187); -x_189 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__4; -lean_inc(x_167); -x_190 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_190, 0, x_167); -lean_ctor_set(x_190, 1, x_189); -x_191 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__5; -lean_inc(x_167); -x_192 = l_Lean_Syntax_node1(x_167, x_191, x_190); -lean_inc(x_167); -x_193 = l_Lean_Syntax_node1(x_167, x_186, x_192); -lean_inc_n(x_188, 4); -x_194 = l_Lean_Syntax_node6(x_167, x_25, x_188, x_188, x_188, x_193, x_188, x_188); -lean_inc(x_1); -x_195 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1(x_19, x_1, x_21, x_22, x_23, x_194, x_6, x_7, x_185); -lean_dec(x_19); -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_12 = x_196; -x_13 = x_197; -goto block_18; +lean_object* x_18; lean_object* x_19; +x_18 = lean_ctor_get(x_15, 1); +lean_inc(x_18); +lean_dec(x_15); +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_13); +lean_ctor_set(x_19, 1, x_18); +return x_19; } } else { -lean_object* x_198; lean_object* x_199; lean_object* x_200; -lean_dec(x_23); -lean_dec(x_22); -lean_dec(x_21); -lean_dec(x_19); -x_198 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_198, 0, x_141); -x_199 = lean_box(0); -lean_inc(x_7); -lean_inc(x_6); -x_200 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__5(x_20, x_25, x_24, x_199, x_198, x_6, x_7, x_8); -lean_dec(x_20); -if (lean_obj_tag(x_200) == 0) +uint8_t x_20; +lean_dec(x_13); +x_20 = !lean_is_exclusive(x_15); +if (x_20 == 0) { -lean_object* x_201; lean_object* x_202; -x_201 = lean_ctor_get(x_200, 0); -lean_inc(x_201); -x_202 = lean_ctor_get(x_200, 1); -lean_inc(x_202); -lean_dec(x_200); -x_12 = x_201; -x_13 = x_202; -goto block_18; +return x_15; +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_15, 0); +x_22 = lean_ctor_get(x_15, 1); +lean_inc(x_22); +lean_inc(x_21); +lean_dec(x_15); +x_23 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_23, 0, x_21); +lean_ctor_set(x_23, 1, x_22); +return x_23; +} +} } else { -uint8_t x_203; +uint8_t x_24; +lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_1); -x_203 = !lean_is_exclusive(x_200); -if (x_203 == 0) +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_24 = !lean_is_exclusive(x_12); +if (x_24 == 0) { -return x_200; +return x_12; } else { -lean_object* x_204; lean_object* x_205; lean_object* x_206; -x_204 = lean_ctor_get(x_200, 0); -x_205 = lean_ctor_get(x_200, 1); -lean_inc(x_205); -lean_inc(x_204); -lean_dec(x_200); -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; +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_EXPORT lean_object* l_Lean_Elab_Command_elabInductives(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_alloc_closure((void*)(l_Lean_Elab_Command_elabInductives___lambda__1), 9, 1); +lean_closure_set(x_5, 0, x_1); +x_6 = l_Lean_Elab_Command_runTermElabM___rarg(x_5, x_2, x_3, x_4); +if (lean_obj_tag(x_6) == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_6, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_6, 1); +lean_inc(x_8); +lean_dec(x_6); +x_9 = l_Lean_Elab_Command_elabInductiveViewsPostprocessing(x_7, x_2, x_3, x_8); +return x_9; } else { -lean_object* x_207; lean_object* x_208; lean_object* x_209; -lean_dec(x_83); -lean_dec(x_23); -lean_dec(x_22); -lean_dec(x_21); -lean_dec(x_19); -x_207 = lean_box(0); -x_208 = lean_box(0); -lean_inc(x_7); -lean_inc(x_6); -x_209 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__5(x_20, x_25, x_24, x_208, x_207, x_6, x_7, x_8); -lean_dec(x_20); -if (lean_obj_tag(x_209) == 0) +uint8_t x_10; +lean_dec(x_3); +lean_dec(x_2); +x_10 = !lean_is_exclusive(x_6); +if (x_10 == 0) { -lean_object* x_210; lean_object* x_211; -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_12 = x_210; -x_13 = x_211; -goto block_18; +return x_6; } else { -uint8_t x_212; -lean_dec(x_7); +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_6, 0); +x_12 = lean_ctor_get(x_6, 1); +lean_inc(x_12); +lean_inc(x_11); lean_dec(x_6); -lean_dec(x_5); +x_13 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_13, 0, x_11); +lean_ctor_set(x_13, 1, x_12); +return x_13; +} +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabInductives___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_212 = !lean_is_exclusive(x_209); -if (x_212 == 0) +x_12 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_13 = l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabInductives___spec__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_Lean_Elab_Command_elabInductive(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: { -return x_209; +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_6 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_6, 0, x_1); +lean_ctor_set(x_6, 1, x_2); +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_array_mk(x_8); +x_10 = l_Lean_Elab_Command_elabInductives(x_9, x_3, x_4, x_5); +return x_10; } -else +} +static lean_object* _init_l_Lean_Elab_Command_elabClassInductive___closed__1() { +_start: { -lean_object* x_213; lean_object* x_214; lean_object* x_215; -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_alloc_ctor(1, 2, 0); -lean_ctor_set(x_215, 0, x_213); -lean_ctor_set(x_215, 1, x_214); -return x_215; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("class", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabClassInductive___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Command_elabClassInductive___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } +static lean_object* _init_l_Lean_Elab_Command_elabClassInductive___closed__3() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = 0; +x_2 = l_Lean_Elab_Command_elabClassInductive___closed__2; +x_3 = lean_box(0); +x_4 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_4, 0, x_2); +lean_ctor_set(x_4, 1, x_3); +lean_ctor_set_uint8(x_4, sizeof(void*)*2, x_1); +return x_4; } } +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabClassInductive(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_Elab_Command_elabClassInductive___closed__3; +x_7 = l_Lean_Elab_Modifiers_addAttr(x_1, x_6); +x_8 = l_Lean_Elab_Command_elabInductive(x_7, x_2, x_3, x_4, x_5); +return x_8; } } +static lean_object* _init_l_Array_anyMUnsafe_any___at_Lean_Elab_Command_isMutualInductive___spec__1___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; +x_2 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__1; +x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__7; +x_4 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__2; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__2(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Command_isMutualInductive___spec__1(lean_object* x_1, size_t x_2, size_t x_3) { _start: { -uint8_t x_5; -x_5 = lean_usize_dec_lt(x_3, x_2); -if (x_5 == 0) +uint8_t x_4; +x_4 = lean_usize_dec_eq(x_2, x_3); +if (x_4 == 0) { -lean_dec(x_1); -return 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; +x_5 = lean_array_uget(x_1, x_2); +x_6 = lean_unsigned_to_nat(1u); +x_7 = l_Lean_Syntax_getArg(x_5, x_6); +lean_dec(x_5); +x_8 = l_Lean_Syntax_getKind(x_7); +x_9 = l_Array_anyMUnsafe_any___at_Lean_Elab_Command_isMutualInductive___spec__1___closed__1; +x_10 = lean_name_eq(x_8, x_9); +lean_dec(x_8); +if (x_10 == 0) +{ +uint8_t x_11; +x_11 = 1; +return x_11; } else { -lean_object* x_6; lean_object* x_7; lean_object* x_8; size_t x_9; size_t x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_6 = lean_array_uget(x_4, x_3); -x_7 = lean_unsigned_to_nat(0u); -x_8 = lean_array_uset(x_4, x_3, x_7); -x_9 = 1; -x_10 = lean_usize_add(x_3, x_9); -x_11 = lean_ctor_get(x_6, 2); -lean_inc(x_11); -lean_dec(x_6); -lean_inc(x_1); -x_12 = l_Lean_Name_append(x_1, x_11); -x_13 = lean_array_uset(x_8, x_3, x_12); -x_3 = x_10; -x_4 = x_13; +size_t x_12; size_t x_13; +x_12 = 1; +x_13 = lean_usize_add(x_2, x_12); +x_2 = x_13; goto _start; } } +else +{ +uint8_t x_15; +x_15 = 0; +return x_15; +} +} } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___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_EXPORT uint8_t l_Lean_Elab_Command_isMutualInductive(lean_object* x_1) { _start: { -uint8_t x_8; -x_8 = lean_usize_dec_lt(x_3, x_2); -if (x_8 == 0) +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; uint8_t x_7; +x_2 = lean_unsigned_to_nat(1u); +x_3 = l_Lean_Syntax_getArg(x_1, x_2); +x_4 = l_Lean_Syntax_getArgs(x_3); +lean_dec(x_3); +x_5 = lean_array_get_size(x_4); +x_6 = lean_unsigned_to_nat(0u); +x_7 = lean_nat_dec_lt(x_6, x_5); +if (x_7 == 0) { -lean_object* x_9; -lean_dec(x_6); +uint8_t x_8; 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_12; lean_object* x_13; lean_object* x_14; size_t x_15; size_t x_16; lean_object* x_17; -x_10 = lean_array_uget(x_1, x_3); -x_11 = lean_ctor_get(x_10, 4); -lean_inc(x_11); -x_12 = lean_ctor_get(x_10, 10); -lean_inc(x_12); -lean_dec(x_10); -x_13 = lean_ctor_get(x_4, 0); -lean_inc(x_13); -x_14 = lean_ctor_get(x_4, 1); -lean_inc(x_14); lean_dec(x_4); -x_15 = lean_array_size(x_12); -x_16 = 0; -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_11); -x_17 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1(x_11, x_12, x_15, x_16, x_13, x_5, x_6, x_7); -if (lean_obj_tag(x_17) == 0) -{ -lean_object* x_18; lean_object* x_19; size_t x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; size_t x_25; size_t x_26; -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_17, 1); -lean_inc(x_19); -lean_dec(x_17); -x_20 = lean_array_size(x_12); -lean_inc(x_11); -x_21 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__2(x_11, x_20, x_16, x_12); -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_11); -lean_ctor_set(x_22, 1, x_21); -x_23 = lean_array_push(x_14, x_22); -x_24 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_24, 0, x_18); -lean_ctor_set(x_24, 1, x_23); -x_25 = 1; -x_26 = lean_usize_add(x_3, x_25); -x_3 = x_26; -x_4 = x_24; -x_7 = x_19; -goto _start; +x_8 = 1; +return x_8; } else { -uint8_t x_28; -lean_dec(x_14); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_6); +size_t x_9; size_t x_10; uint8_t x_11; +x_9 = 0; +x_10 = lean_usize_of_nat(x_5); lean_dec(x_5); -x_28 = !lean_is_exclusive(x_17); -if (x_28 == 0) +x_11 = l_Array_anyMUnsafe_any___at_Lean_Elab_Command_isMutualInductive___spec__1(x_4, x_9, x_10); +lean_dec(x_4); +if (x_11 == 0) { -return x_17; +uint8_t x_12; +x_12 = 1; +return x_12; } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_17, 0); -x_30 = lean_ctor_get(x_17, 1); -lean_inc(x_30); -lean_inc(x_29); -lean_dec(x_17); -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; +uint8_t x_13; +x_13 = 0; +return x_13; } } } } +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Command_isMutualInductive___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; size_t x_5; uint8_t x_6; lean_object* x_7; +x_4 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_5 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_6 = l_Array_anyMUnsafe_any___at_Lean_Elab_Command_isMutualInductive___spec__1(x_1, x_4, x_5); +lean_dec(x_1); +x_7 = lean_box(x_6); +return x_7; +} } -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__4(lean_object* x_1, size_t x_2, size_t x_3) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_isMutualInductive___boxed(lean_object* x_1) { _start: { -uint8_t x_4; -x_4 = lean_usize_dec_eq(x_2, x_3); -if (x_4 == 0) +uint8_t x_2; lean_object* x_3; +x_2 = l_Lean_Elab_Command_isMutualInductive(x_1); +lean_dec(x_1); +x_3 = lean_box(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabMutualInductive___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; uint8_t x_7; -x_5 = lean_array_uget(x_1, x_2); -x_6 = lean_ctor_get(x_5, 10); +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_5 = l_Lean_Elab_Command_getRef(x_2, x_3, x_4); +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_7 = l_Array_isEmpty___rarg(x_6); +x_8 = lean_ctor_get(x_2, 4); +lean_inc(x_8); +lean_inc(x_8); +x_9 = l_Lean_Elab_getBetterRef(x_6, x_8); lean_dec(x_6); -if (x_7 == 0) +x_10 = l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1(x_1, x_2, x_3, x_7); +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) { -uint8_t x_8; -x_8 = 1; -return x_8; +lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_12 = lean_ctor_get(x_10, 0); +x_13 = lean_ctor_get(x_10, 1); +x_14 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_12, x_8, x_2, x_3, x_13); +lean_dec(x_2); +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 0) +{ +lean_object* x_16; +x_16 = lean_ctor_get(x_14, 0); +lean_ctor_set(x_10, 1, x_16); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set_tag(x_14, 1); +lean_ctor_set(x_14, 0, x_10); +return x_14; } else { -size_t x_9; size_t x_10; -x_9 = 1; -x_10 = lean_usize_add(x_2, x_9); -x_2 = x_10; -goto _start; +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_14, 0); +x_18 = lean_ctor_get(x_14, 1); +lean_inc(x_18); +lean_inc(x_17); +lean_dec(x_14); +lean_ctor_set(x_10, 1, x_17); +lean_ctor_set(x_10, 0, x_9); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_10); +lean_ctor_set(x_19, 1, x_18); +return x_19; } } else { -uint8_t x_12; -x_12 = 0; -return x_12; +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_20 = lean_ctor_get(x_10, 0); +x_21 = lean_ctor_get(x_10, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_10); +x_22 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_20, x_8, x_2, x_3, x_21); +lean_dec(x_2); +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +if (lean_is_exclusive(x_22)) { + lean_ctor_release(x_22, 0); + lean_ctor_release(x_22, 1); + x_25 = x_22; +} else { + lean_dec_ref(x_22); + x_25 = lean_box(0); } +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_9); +lean_ctor_set(x_26, 1, x_23); +if (lean_is_scalar(x_25)) { + x_27 = lean_alloc_ctor(1, 2, 0); +} else { + x_27 = x_25; + lean_ctor_set_tag(x_27, 1); } +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_24); +return x_27; } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__1___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("genMatcherCode", 14, 14); -return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__1___closed__2() { +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabMutualInductive___spec__7(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_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__1; -x_2 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__1___closed__1; -x_3 = l_Lean_Name_mkStr2(x_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; uint8_t x_11; +x_5 = l_Lean_Elab_Command_getRef(x_2, x_3, x_4); +x_6 = lean_ctor_get(x_5, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_5, 1); +lean_inc(x_7); +lean_dec(x_5); +x_8 = lean_ctor_get(x_2, 4); +lean_inc(x_8); +lean_inc(x_8); +x_9 = l_Lean_Elab_getBetterRef(x_6, x_8); +lean_dec(x_6); +x_10 = l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1(x_1, x_2, x_3, x_7); +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_12 = lean_ctor_get(x_10, 0); +x_13 = lean_ctor_get(x_10, 1); +x_14 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_12, x_8, x_2, x_3, x_13); +lean_dec(x_2); +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 0) +{ +lean_object* x_16; +x_16 = lean_ctor_get(x_14, 0); +lean_ctor_set(x_10, 1, x_16); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set_tag(x_14, 1); +lean_ctor_set(x_14, 0, x_10); +return x_14; } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__1___closed__3() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("elaboratingComputedFields", 25, 25); -return x_1; +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_14, 0); +x_18 = lean_ctor_get(x_14, 1); +lean_inc(x_18); +lean_inc(x_17); +lean_dec(x_14); +lean_ctor_set(x_10, 1, x_17); +lean_ctor_set(x_10, 0, x_9); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_10); +lean_ctor_set(x_19, 1, x_18); +return x_19; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__1___closed__4() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__1___closed__3; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_20 = lean_ctor_get(x_10, 0); +x_21 = lean_ctor_get(x_10, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_10); +x_22 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_20, x_8, x_2, x_3, x_21); +lean_dec(x_2); +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +if (lean_is_exclusive(x_22)) { + lean_ctor_release(x_22, 0); + lean_ctor_release(x_22, 1); + x_25 = x_22; +} else { + lean_dec_ref(x_22); + x_25 = lean_box(0); +} +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_9); +lean_ctor_set(x_26, 1, x_23); +if (lean_is_scalar(x_25)) { + x_27 = lean_alloc_ctor(1, 2, 0); +} else { + x_27 = x_25; + lean_ctor_set_tag(x_27, 1); } +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_24); +return x_27; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__1(lean_object* x_1) { +} +} +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabMutualInductive___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -uint8_t x_2; -x_2 = !lean_is_exclusive(x_1); -if (x_2 == 0) +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; +x_6 = l_Lean_Elab_Command_getRef(x_3, x_4, x_5); +x_7 = lean_ctor_get(x_6, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_6, 1); +lean_inc(x_8); +lean_dec(x_6); +x_9 = l_Lean_replaceRef(x_1, x_7); +lean_dec(x_7); +x_10 = !lean_is_exclusive(x_3); +if (x_10 == 0) { -lean_object* x_3; lean_object* x_4; uint8_t x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; lean_object* x_9; -x_3 = lean_ctor_get(x_1, 1); -x_4 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__1___closed__2; -x_5 = 0; -x_6 = l_Lean_KVMap_setBool(x_3, x_4, x_5); -x_7 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__1___closed__4; -x_8 = 1; -x_9 = l_Lean_KVMap_setBool(x_6, x_7, x_8); -lean_ctor_set(x_1, 1, x_9); -return x_1; +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_elabMutualInductive___spec__7(x_2, x_3, x_4, x_8); +return x_12; } 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; uint8_t x_19; lean_object* x_20; uint8_t x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; lean_object* x_25; lean_object* x_26; -x_10 = lean_ctor_get(x_1, 0); -x_11 = lean_ctor_get(x_1, 1); -x_12 = lean_ctor_get(x_1, 2); -x_13 = lean_ctor_get(x_1, 3); -x_14 = lean_ctor_get(x_1, 4); -x_15 = lean_ctor_get(x_1, 5); -x_16 = lean_ctor_get(x_1, 6); -x_17 = lean_ctor_get(x_1, 7); -x_18 = lean_ctor_get(x_1, 8); -x_19 = lean_ctor_get_uint8(x_1, sizeof(void*)*9); +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; lean_object* x_24; +x_13 = lean_ctor_get(x_3, 0); +x_14 = lean_ctor_get(x_3, 1); +x_15 = lean_ctor_get(x_3, 2); +x_16 = lean_ctor_get(x_3, 3); +x_17 = lean_ctor_get(x_3, 4); +x_18 = lean_ctor_get(x_3, 5); +x_19 = lean_ctor_get(x_3, 7); +x_20 = lean_ctor_get(x_3, 8); +x_21 = lean_ctor_get(x_3, 9); +x_22 = lean_ctor_get_uint8(x_3, sizeof(void*)*10); +lean_inc(x_21); +lean_inc(x_20); +lean_inc(x_19); lean_inc(x_18); lean_inc(x_17); lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_dec(x_1); -x_20 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__1___closed__2; -x_21 = 0; -x_22 = l_Lean_KVMap_setBool(x_11, x_20, x_21); -x_23 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__1___closed__4; -x_24 = 1; -x_25 = l_Lean_KVMap_setBool(x_22, x_23, x_24); -x_26 = lean_alloc_ctor(0, 9, 1); -lean_ctor_set(x_26, 0, x_10); -lean_ctor_set(x_26, 1, x_25); -lean_ctor_set(x_26, 2, x_12); -lean_ctor_set(x_26, 3, x_13); -lean_ctor_set(x_26, 4, x_14); -lean_ctor_set(x_26, 5, x_15); -lean_ctor_set(x_26, 6, x_16); -lean_ctor_set(x_26, 7, x_17); -lean_ctor_set(x_26, 8, x_18); -lean_ctor_set_uint8(x_26, sizeof(void*)*9, x_19); -return x_26; +lean_dec(x_3); +x_23 = lean_alloc_ctor(0, 10, 1); +lean_ctor_set(x_23, 0, x_13); +lean_ctor_set(x_23, 1, x_14); +lean_ctor_set(x_23, 2, x_15); +lean_ctor_set(x_23, 3, x_16); +lean_ctor_set(x_23, 4, x_17); +lean_ctor_set(x_23, 5, x_18); +lean_ctor_set(x_23, 6, x_9); +lean_ctor_set(x_23, 7, x_19); +lean_ctor_set(x_23, 8, x_20); +lean_ctor_set(x_23, 9, x_21); +lean_ctor_set_uint8(x_23, sizeof(void*)*10, x_22); +x_24 = l_Lean_throwError___at_Lean_Elab_Command_elabMutualInductive___spec__7(x_2, x_23, x_4, x_8); +return x_24; } } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualInductive___spec__4___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) { _start: { -lean_object* x_9; -x_9 = l_Lean_Elab_ComputedFields_setComputedFields(x_1, x_4, x_5, x_6, x_7, x_8); -return x_9; -} -} -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__1() { -_start: +lean_object* x_7; uint8_t x_8; +x_7 = lean_st_ref_get(x_5, x_6); +x_8 = !lean_is_exclusive(x_7); +if (x_8 == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_9 = lean_ctor_get(x_7, 0); +x_10 = lean_ctor_get(x_7, 1); +x_11 = lean_ctor_get(x_9, 0); +lean_inc(x_11); +lean_dec(x_9); +lean_inc(x_3); +x_12 = l_Lean_getAttributeImpl(x_11, x_3); +lean_dec(x_11); +if (lean_obj_tag(x_12) == 0) { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__3___closed__1; -x_2 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_2, 0, x_1); -lean_ctor_set(x_2, 1, x_1); -return x_2; -} +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +lean_dec(x_12); +lean_free_object(x_7); +lean_dec(x_2); +x_13 = l_Lean_MessageData_ofName(x_3); +x_14 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__2___closed__2; +x_15 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_13); +x_16 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__2___closed__4; +x_17 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_17, 0, x_15); +lean_ctor_set(x_17, 1, x_16); +x_18 = l_Lean_throwError___at_Lean_Elab_Command_elabMutualInductive___spec__5(x_17, x_4, x_5, x_10); +return x_18; } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__2() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("mutual", 6, 6); -return x_1; +lean_object* x_19; +lean_dec(x_12); +lean_dec(x_4); +x_19 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_19, 0, x_3); +lean_ctor_set(x_19, 1, x_2); +lean_ctor_set_uint8(x_19, sizeof(void*)*2, x_1); +lean_ctor_set(x_7, 0, x_19); +return x_7; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__3() { -_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_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__4; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__1; -x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__7; -x_4 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__2; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; -} +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_20 = lean_ctor_get(x_7, 0); +x_21 = lean_ctor_get(x_7, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_7); +x_22 = lean_ctor_get(x_20, 0); +lean_inc(x_22); +lean_dec(x_20); +lean_inc(x_3); +x_23 = l_Lean_getAttributeImpl(x_22, x_3); +lean_dec(x_22); +if (lean_obj_tag(x_23) == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +lean_dec(x_23); +lean_dec(x_2); +x_24 = l_Lean_MessageData_ofName(x_3); +x_25 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__2___closed__2; +x_26 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_24); +x_27 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__2___closed__4; +x_28 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +x_29 = l_Lean_throwError___at_Lean_Elab_Command_elabMutualInductive___spec__5(x_28, x_4, x_5, x_21); +return x_29; } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__4() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("end", 3, 3); -return x_1; +lean_object* x_30; lean_object* x_31; +lean_dec(x_23); +lean_dec(x_4); +x_30 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_30, 0, x_3); +lean_ctor_set(x_30, 1, x_2); +lean_ctor_set_uint8(x_30, sizeof(void*)*2, x_1); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_30); +lean_ctor_set(x_31, 1, x_21); +return x_31; } } -static lean_object* _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__5() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__1), 1, 0); -return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualInductive___spec__4(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; lean_object* x_9; -x_6 = lean_array_size(x_1); -x_7 = 0; -x_8 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__1; -lean_inc(x_4); -lean_inc(x_3); -x_9 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__3(x_1, x_6, x_7, x_8, x_3, x_4, x_5); -if (lean_obj_tag(x_9) == 0) +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Lean_Syntax_getArg(x_1, x_5); +x_7 = lean_alloc_closure((void*)(l_Lean_Elab_toAttributeKind___boxed), 3, 1); +lean_closure_set(x_7, 0, x_6); +lean_inc(x_2); +x_8 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_mkDefViewOfInstance___spec__1(x_7, x_2, x_3, x_4); +if (lean_obj_tag(x_8) == 0) { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; -x_10 = lean_ctor_get(x_9, 0); +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_9 = lean_ctor_get(x_8, 0); +lean_inc(x_9); +x_10 = lean_ctor_get(x_8, 1); lean_inc(x_10); -x_11 = lean_ctor_get(x_9, 1); -lean_inc(x_11); -lean_dec(x_9); -x_12 = lean_ctor_get(x_10, 0); -lean_inc(x_12); -x_13 = lean_ctor_get(x_10, 1); -lean_inc(x_13); -lean_dec(x_10); -x_14 = l_Lean_Elab_Command_getRef(x_3, x_4, x_11); -x_15 = lean_ctor_get(x_14, 0); -lean_inc(x_15); -x_16 = lean_ctor_get(x_14, 1); +lean_dec(x_8); +x_11 = lean_unsigned_to_nat(1u); +x_12 = l_Lean_Syntax_getArg(x_1, x_11); +x_13 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__1; +x_14 = lean_alloc_closure((void*)(l_Lean_expandMacros), 4, 2); +lean_closure_set(x_14, 0, x_12); +lean_closure_set(x_14, 1, x_13); +lean_inc(x_2); +x_15 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__13(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; +x_16 = lean_ctor_get(x_15, 0); lean_inc(x_16); -lean_dec(x_14); -x_17 = 0; -x_18 = l_Lean_SourceInfo_fromRef(x_15, x_17); +x_17 = lean_ctor_get(x_15, 1); +lean_inc(x_17); lean_dec(x_15); -x_19 = l_Lean_Elab_Command_getCurrMacroScope(x_3, x_4, x_16); -x_20 = !lean_is_exclusive(x_19); +lean_inc(x_16); +x_18 = l_Lean_Syntax_getKind(x_16); +x_19 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__4; +x_20 = lean_name_eq(x_18, x_19); if (x_20 == 0) { -lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; -x_21 = lean_ctor_get(x_19, 1); -x_22 = lean_ctor_get(x_19, 0); -lean_dec(x_22); -x_23 = l_Lean_Elab_Command_getMainModule___rarg(x_4, x_21); -x_24 = !lean_is_exclusive(x_23); -if (x_24 == 0) +if (lean_obj_tag(x_18) == 1) { -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_23, 1); -x_26 = lean_ctor_get(x_23, 0); -lean_dec(x_26); -x_27 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__2; -lean_inc(x_18); -lean_ctor_set_tag(x_23, 2); -lean_ctor_set(x_23, 1, x_27); -lean_ctor_set(x_23, 0, x_18); -x_28 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; -x_29 = l_Array_append___rarg(x_28, x_12); -lean_dec(x_12); -x_30 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__12; -lean_inc(x_18); -x_31 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_31, 0, x_18); -lean_ctor_set(x_31, 1, x_30); -lean_ctor_set(x_31, 2, x_29); -x_32 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__4; -lean_inc(x_18); -lean_ctor_set_tag(x_19, 2); -lean_ctor_set(x_19, 1, x_32); -lean_ctor_set(x_19, 0, x_18); -x_33 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__3; -x_34 = l_Lean_Syntax_node3(x_18, x_33, x_23, x_31, x_19); -x_35 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabCommand), 4, 1); -lean_closure_set(x_35, 0, x_34); -x_36 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__5; -lean_inc(x_4); -lean_inc(x_3); -x_37 = l_Lean_Elab_Command_withScope___rarg(x_36, x_35, x_3, x_4, x_25); -if (lean_obj_tag(x_37) == 0) +lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; lean_object* x_25; +x_21 = lean_ctor_get(x_18, 1); +lean_inc(x_21); +lean_dec(x_18); +x_22 = lean_box(0); +x_23 = l_Lean_Name_str___override(x_22, x_21); +x_24 = lean_unbox(x_9); +lean_dec(x_9); +x_25 = l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualInductive___spec__4___lambda__1(x_24, x_16, x_23, x_2, x_3, x_17); +return x_25; +} +else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; lean_object* x_42; -x_38 = lean_ctor_get(x_37, 1); -lean_inc(x_38); -lean_dec(x_37); -x_39 = lean_array_get_size(x_1); -x_40 = lean_unsigned_to_nat(0u); -x_41 = lean_nat_dec_lt(x_40, x_39); -lean_dec(x_39); -x_42 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__2___boxed), 8, 1); -lean_closure_set(x_42, 0, x_13); -if (x_41 == 0) +lean_object* x_26; lean_object* x_27; uint8_t x_28; +lean_dec(x_18); +lean_dec(x_9); +x_26 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__6; +x_27 = l_Lean_throwErrorAt___at_Lean_Elab_Command_elabMutualInductive___spec__6(x_16, x_26, x_2, x_3, x_17); +lean_dec(x_16); +x_28 = !lean_is_exclusive(x_27); +if (x_28 == 0) { -lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_43 = l_Lean_Elab_Command_instInhabitedInductiveView; -x_44 = l_outOfBounds___rarg(x_43); -x_45 = lean_ctor_get(x_44, 4); -lean_inc(x_45); -lean_dec(x_44); -x_46 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withDeclName___rarg), 9, 2); -lean_closure_set(x_46, 0, x_45); -lean_closure_set(x_46, 1, x_42); -x_47 = l_Lean_Elab_Command_liftTermElabM___rarg(x_46, x_3, x_4, x_38); -lean_dec(x_4); -lean_dec(x_3); -return x_47; +return x_27; } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_48 = lean_array_fget(x_1, x_40); -x_49 = lean_ctor_get(x_48, 4); -lean_inc(x_49); -lean_dec(x_48); -x_50 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withDeclName___rarg), 9, 2); -lean_closure_set(x_50, 0, x_49); -lean_closure_set(x_50, 1, x_42); -x_51 = l_Lean_Elab_Command_liftTermElabM___rarg(x_50, x_3, x_4, x_38); -lean_dec(x_4); -lean_dec(x_3); -return x_51; +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_27, 0); +x_30 = lean_ctor_get(x_27, 1); +lean_inc(x_30); +lean_inc(x_29); +lean_dec(x_27); +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_52; -lean_dec(x_13); -lean_dec(x_4); -lean_dec(x_3); -x_52 = !lean_is_exclusive(x_37); -if (x_52 == 0) -{ -return x_37; } else { -lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_53 = lean_ctor_get(x_37, 0); -x_54 = lean_ctor_get(x_37, 1); -lean_inc(x_54); -lean_inc(x_53); -lean_dec(x_37); -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_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; lean_object* x_36; +lean_dec(x_18); +x_32 = l_Lean_Syntax_getArg(x_16, x_5); +x_33 = l_Lean_Syntax_getId(x_32); +lean_dec(x_32); +x_34 = lean_erase_macro_scopes(x_33); +x_35 = lean_unbox(x_9); +lean_dec(x_9); +x_36 = l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualInductive___spec__4___lambda__1(x_35, x_16, x_34, x_2, x_3, x_17); +return x_36; } } else { -lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_56 = lean_ctor_get(x_23, 1); -lean_inc(x_56); -lean_dec(x_23); -x_57 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__2; -lean_inc(x_18); -x_58 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_58, 0, x_18); -lean_ctor_set(x_58, 1, x_57); -x_59 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; -x_60 = l_Array_append___rarg(x_59, x_12); -lean_dec(x_12); -x_61 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__12; -lean_inc(x_18); -x_62 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_62, 0, x_18); -lean_ctor_set(x_62, 1, x_61); -lean_ctor_set(x_62, 2, x_60); -x_63 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__4; -lean_inc(x_18); -lean_ctor_set_tag(x_19, 2); -lean_ctor_set(x_19, 1, x_63); -lean_ctor_set(x_19, 0, x_18); -x_64 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__3; -x_65 = l_Lean_Syntax_node3(x_18, x_64, x_58, x_62, x_19); -x_66 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabCommand), 4, 1); -lean_closure_set(x_66, 0, x_65); -x_67 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__5; -lean_inc(x_4); -lean_inc(x_3); -x_68 = l_Lean_Elab_Command_withScope___rarg(x_67, x_66, x_3, x_4, x_56); -if (lean_obj_tag(x_68) == 0) -{ -lean_object* x_69; lean_object* x_70; lean_object* x_71; uint8_t x_72; lean_object* x_73; -x_69 = lean_ctor_get(x_68, 1); -lean_inc(x_69); -lean_dec(x_68); -x_70 = lean_array_get_size(x_1); -x_71 = lean_unsigned_to_nat(0u); -x_72 = lean_nat_dec_lt(x_71, x_70); -lean_dec(x_70); -x_73 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__2___boxed), 8, 1); -lean_closure_set(x_73, 0, x_13); -if (x_72 == 0) +uint8_t x_37; +lean_dec(x_9); +lean_dec(x_2); +x_37 = !lean_is_exclusive(x_15); +if (x_37 == 0) { -lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; -x_74 = l_Lean_Elab_Command_instInhabitedInductiveView; -x_75 = l_outOfBounds___rarg(x_74); -x_76 = lean_ctor_get(x_75, 4); -lean_inc(x_76); -lean_dec(x_75); -x_77 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withDeclName___rarg), 9, 2); -lean_closure_set(x_77, 0, x_76); -lean_closure_set(x_77, 1, x_73); -x_78 = l_Lean_Elab_Command_liftTermElabM___rarg(x_77, x_3, x_4, x_69); -lean_dec(x_4); -lean_dec(x_3); -return x_78; +return x_15; } else { -lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; -x_79 = lean_array_fget(x_1, x_71); -x_80 = lean_ctor_get(x_79, 4); -lean_inc(x_80); -lean_dec(x_79); -x_81 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withDeclName___rarg), 9, 2); -lean_closure_set(x_81, 0, x_80); -lean_closure_set(x_81, 1, x_73); -x_82 = l_Lean_Elab_Command_liftTermElabM___rarg(x_81, x_3, x_4, x_69); -lean_dec(x_4); -lean_dec(x_3); -return x_82; +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_15, 0); +x_39 = lean_ctor_get(x_15, 1); +lean_inc(x_39); +lean_inc(x_38); +lean_dec(x_15); +x_40 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +return x_40; +} } } else { -lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; -lean_dec(x_13); -lean_dec(x_4); -lean_dec(x_3); -x_83 = lean_ctor_get(x_68, 0); -lean_inc(x_83); -x_84 = lean_ctor_get(x_68, 1); -lean_inc(x_84); -if (lean_is_exclusive(x_68)) { - lean_ctor_release(x_68, 0); - lean_ctor_release(x_68, 1); - x_85 = x_68; -} else { - lean_dec_ref(x_68); - x_85 = lean_box(0); +uint8_t x_41; +lean_dec(x_2); +x_41 = !lean_is_exclusive(x_8); +if (x_41 == 0) +{ +return x_8; +} +else +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_42 = lean_ctor_get(x_8, 0); +x_43 = lean_ctor_get(x_8, 1); +lean_inc(x_43); +lean_inc(x_42); +lean_dec(x_8); +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; } -if (lean_is_scalar(x_85)) { - x_86 = lean_alloc_ctor(1, 2, 0); -} else { - x_86 = x_85; } -lean_ctor_set(x_86, 0, x_83); -lean_ctor_set(x_86, 1, x_84); -return x_86; } } +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabMutualInductive___spec__8(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_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_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_87 = lean_ctor_get(x_19, 1); -lean_inc(x_87); +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; lean_object* x_32; lean_object* x_33; +x_10 = lean_array_uget(x_1, x_3); +x_18 = l_Lean_Elab_Command_getRef(x_5, x_6, x_7); +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_replaceRef(x_10, x_19); lean_dec(x_19); -x_88 = l_Lean_Elab_Command_getMainModule___rarg(x_4, x_87); -x_89 = lean_ctor_get(x_88, 1); -lean_inc(x_89); -if (lean_is_exclusive(x_88)) { - lean_ctor_release(x_88, 0); - lean_ctor_release(x_88, 1); - x_90 = x_88; -} else { - lean_dec_ref(x_88); - x_90 = lean_box(0); -} -x_91 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__2; -lean_inc(x_18); -if (lean_is_scalar(x_90)) { - x_92 = lean_alloc_ctor(2, 2, 0); -} else { - x_92 = x_90; - lean_ctor_set_tag(x_92, 2); +x_22 = lean_ctor_get(x_5, 0); +lean_inc(x_22); +x_23 = lean_ctor_get(x_5, 1); +lean_inc(x_23); +x_24 = lean_ctor_get(x_5, 2); +lean_inc(x_24); +x_25 = lean_ctor_get(x_5, 3); +lean_inc(x_25); +x_26 = lean_ctor_get(x_5, 4); +lean_inc(x_26); +x_27 = lean_ctor_get(x_5, 5); +lean_inc(x_27); +x_28 = lean_ctor_get(x_5, 7); +lean_inc(x_28); +x_29 = lean_ctor_get(x_5, 8); +lean_inc(x_29); +x_30 = lean_ctor_get(x_5, 9); +lean_inc(x_30); +x_31 = lean_ctor_get_uint8(x_5, sizeof(void*)*10); +x_32 = lean_alloc_ctor(0, 10, 1); +lean_ctor_set(x_32, 0, x_22); +lean_ctor_set(x_32, 1, x_23); +lean_ctor_set(x_32, 2, x_24); +lean_ctor_set(x_32, 3, x_25); +lean_ctor_set(x_32, 4, x_26); +lean_ctor_set(x_32, 5, x_27); +lean_ctor_set(x_32, 6, x_21); +lean_ctor_set(x_32, 7, x_28); +lean_ctor_set(x_32, 8, x_29); +lean_ctor_set(x_32, 9, x_30); +lean_ctor_set_uint8(x_32, sizeof(void*)*10, x_31); +x_33 = l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualInductive___spec__4(x_10, x_32, x_6, x_20); +lean_dec(x_10); +if (lean_obj_tag(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_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_push(x_4, x_34); +x_37 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_37, 0, x_36); +x_11 = x_37; +x_12 = x_35; +goto block_17; } -lean_ctor_set(x_92, 0, x_18); -lean_ctor_set(x_92, 1, x_91); -x_93 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; -x_94 = l_Array_append___rarg(x_93, x_12); -lean_dec(x_12); -x_95 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__12; -lean_inc(x_18); -x_96 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_96, 0, x_18); -lean_ctor_set(x_96, 1, x_95); -lean_ctor_set(x_96, 2, x_94); -x_97 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__4; -lean_inc(x_18); -x_98 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_98, 0, x_18); -lean_ctor_set(x_98, 1, x_97); -x_99 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__3; -x_100 = l_Lean_Syntax_node3(x_18, x_99, x_92, x_96, x_98); -x_101 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabCommand), 4, 1); -lean_closure_set(x_101, 0, x_100); -x_102 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__5; -lean_inc(x_4); -lean_inc(x_3); -x_103 = l_Lean_Elab_Command_withScope___rarg(x_102, x_101, x_3, x_4, x_89); -if (lean_obj_tag(x_103) == 0) +else { -lean_object* x_104; lean_object* x_105; lean_object* x_106; uint8_t x_107; lean_object* x_108; -x_104 = lean_ctor_get(x_103, 1); -lean_inc(x_104); -lean_dec(x_103); -x_105 = lean_array_get_size(x_1); -x_106 = lean_unsigned_to_nat(0u); -x_107 = lean_nat_dec_lt(x_106, x_105); -lean_dec(x_105); -x_108 = lean_alloc_closure((void*)(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__2___boxed), 8, 1); -lean_closure_set(x_108, 0, x_13); -if (x_107 == 0) +uint8_t x_38; +x_38 = !lean_is_exclusive(x_33); +if (x_38 == 0) { -lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; -x_109 = l_Lean_Elab_Command_instInhabitedInductiveView; -x_110 = l_outOfBounds___rarg(x_109); -x_111 = lean_ctor_get(x_110, 4); -lean_inc(x_111); -lean_dec(x_110); -x_112 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withDeclName___rarg), 9, 2); -lean_closure_set(x_112, 0, x_111); -lean_closure_set(x_112, 1, x_108); -x_113 = l_Lean_Elab_Command_liftTermElabM___rarg(x_112, x_3, x_4, x_104); +lean_object* x_39; lean_object* x_40; uint8_t x_41; +x_39 = lean_ctor_get(x_33, 0); +x_40 = lean_ctor_get(x_33, 1); +x_41 = l_Lean_Exception_isInterrupt(x_39); +if (x_41 == 0) +{ +lean_object* x_42; +lean_free_object(x_33); +lean_inc(x_5); +x_42 = l_Lean_Elab_logException___at_Lean_Elab_Command_elabCommand___spec__3(x_39, x_5, x_6, x_40); +if (lean_obj_tag(x_42) == 0) +{ +lean_object* x_43; lean_object* x_44; +x_43 = lean_ctor_get(x_42, 1); +lean_inc(x_43); +lean_dec(x_42); +x_44 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_44, 0, x_4); +x_11 = x_44; +x_12 = x_43; +goto block_17; +} +else +{ +uint8_t x_45; +lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); -return x_113; +x_45 = !lean_is_exclusive(x_42); +if (x_45 == 0) +{ +return x_42; } else { -lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; -x_114 = lean_array_fget(x_1, x_106); -x_115 = lean_ctor_get(x_114, 4); -lean_inc(x_115); -lean_dec(x_114); -x_116 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withDeclName___rarg), 9, 2); -lean_closure_set(x_116, 0, x_115); -lean_closure_set(x_116, 1, x_108); -x_117 = l_Lean_Elab_Command_liftTermElabM___rarg(x_116, x_3, x_4, x_104); +lean_object* x_46; lean_object* x_47; lean_object* x_48; +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_alloc_ctor(1, 2, 0); +lean_ctor_set(x_48, 0, x_46); +lean_ctor_set(x_48, 1, x_47); +return x_48; +} +} +} +else +{ +lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); -return x_117; +return x_33; } } else { -lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; -lean_dec(x_13); +lean_object* x_49; lean_object* x_50; uint8_t 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 = l_Lean_Exception_isInterrupt(x_49); +if (x_51 == 0) +{ +lean_object* x_52; +lean_inc(x_5); +x_52 = l_Lean_Elab_logException___at_Lean_Elab_Command_elabCommand___spec__3(x_49, x_5, x_6, x_50); +if (lean_obj_tag(x_52) == 0) +{ +lean_object* x_53; lean_object* x_54; +x_53 = lean_ctor_get(x_52, 1); +lean_inc(x_53); +lean_dec(x_52); +x_54 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_54, 0, x_4); +x_11 = x_54; +x_12 = x_53; +goto block_17; +} +else +{ +lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; +lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); -x_118 = lean_ctor_get(x_103, 0); -lean_inc(x_118); -x_119 = lean_ctor_get(x_103, 1); -lean_inc(x_119); -if (lean_is_exclusive(x_103)) { - lean_ctor_release(x_103, 0); - lean_ctor_release(x_103, 1); - x_120 = x_103; +x_55 = lean_ctor_get(x_52, 0); +lean_inc(x_55); +x_56 = lean_ctor_get(x_52, 1); +lean_inc(x_56); +if (lean_is_exclusive(x_52)) { + lean_ctor_release(x_52, 0); + lean_ctor_release(x_52, 1); + x_57 = x_52; } else { - lean_dec_ref(x_103); - x_120 = lean_box(0); + lean_dec_ref(x_52); + x_57 = lean_box(0); } -if (lean_is_scalar(x_120)) { - x_121 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_57)) { + x_58 = lean_alloc_ctor(1, 2, 0); } else { - x_121 = x_120; -} -lean_ctor_set(x_121, 0, x_118); -lean_ctor_set(x_121, 1, x_119); -return x_121; + x_58 = x_57; } +lean_ctor_set(x_58, 0, x_55); +lean_ctor_set(x_58, 1, x_56); +return x_58; } } else { -uint8_t x_122; +lean_object* x_59; +lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); -x_122 = !lean_is_exclusive(x_9); -if (x_122 == 0) -{ -return x_9; +x_59 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_59, 0, x_49); +lean_ctor_set(x_59, 1, x_50); +return x_59; } -else +} +} +block_17: { -lean_object* x_123; lean_object* x_124; lean_object* x_125; -x_123 = lean_ctor_get(x_9, 0); -x_124 = lean_ctor_get(x_9, 1); -lean_inc(x_124); -lean_inc(x_123); -lean_dec(x_9); -x_125 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_125, 0, x_123); -lean_ctor_set(x_125, 1, x_124); -return x_125; +lean_object* x_13; size_t x_14; size_t x_15; +x_13 = lean_ctor_get(x_11, 0); +lean_inc(x_13); +lean_dec(x_11); +x_14 = 1; +x_15 = lean_usize_add(x_3, x_14); +x_3 = x_15; +x_4 = x_13; +x_7 = x_12; +goto _start; } } } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_elabAttrs___at_Lean_Elab_Command_elabMutualInductive___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_5; lean_object* x_6; uint8_t x_7; -x_5 = lean_array_get_size(x_1); -x_6 = lean_unsigned_to_nat(0u); -x_7 = lean_nat_dec_lt(x_6, x_5); -if (x_7 == 0) -{ -lean_object* x_8; lean_object* x_9; -lean_dec(x_5); -lean_dec(x_3); -lean_dec(x_2); -x_8 = lean_box(0); -x_9 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_9, 0, x_8); -lean_ctor_set(x_9, 1, x_4); -return x_9; -} -else +size_t x_5; size_t x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_array_size(x_1); +x_6 = 0; +x_7 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__8___closed__1; +x_8 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabMutualInductive___spec__8(x_1, x_5, x_6, x_7, x_2, x_3, x_4); +if (lean_obj_tag(x_8) == 0) { -size_t x_10; size_t x_11; uint8_t x_12; -x_10 = 0; -x_11 = lean_usize_of_nat(x_5); -lean_dec(x_5); -x_12 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__4(x_1, x_10, x_11); -if (x_12 == 0) +uint8_t x_9; +x_9 = !lean_is_exclusive(x_8); +if (x_9 == 0) { -lean_object* x_13; lean_object* x_14; -lean_dec(x_3); -lean_dec(x_2); -x_13 = lean_box(0); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_13); -lean_ctor_set(x_14, 1, x_4); -return x_14; +return x_8; } else { -lean_object* x_15; lean_object* x_16; -x_15 = lean_box(0); -x_16 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3(x_1, x_15, x_2, x_3, x_4); -return x_16; -} +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_8, 0); +x_11 = lean_ctor_get(x_8, 1); +lean_inc(x_11); +lean_inc(x_10); +lean_dec(x_8); +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; } } +else +{ +uint8_t x_13; +x_13 = !lean_is_exclusive(x_8); +if (x_13 == 0) +{ +return x_8; } -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* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +else { -lean_object* x_10; -x_10 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_8, 0); +x_15 = lean_ctor_get(x_8, 1); +lean_inc(x_15); +lean_inc(x_14); lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_1); -return 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; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___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: -{ -lean_object* x_11; -x_11 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___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_7); -lean_dec(x_1); -return x_11; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Elab_elabDeclAttrs___at_Lean_Elab_Command_elabMutualInductive___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_11; -x_11 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_unsigned_to_nat(1u); +x_6 = l_Lean_Syntax_getArg(x_1, x_5); +x_7 = l_Lean_Syntax_getSepArgs(x_6); lean_dec(x_6); -lean_dec(x_1); -return x_11; +x_8 = l_Lean_Elab_elabAttrs___at_Lean_Elab_Command_elabMutualInductive___spec__3(x_7, x_2, x_3, x_4); +lean_dec(x_7); +return x_8; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabMutualInductive___spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_10; -x_10 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +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_5 = l_Lean_Elab_Command_getRef(x_2, x_3, x_4); +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); -lean_dec(x_1); -return x_10; -} -} -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___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: +x_8 = lean_ctor_get(x_2, 4); +lean_inc(x_8); +lean_inc(x_8); +x_9 = l_Lean_Elab_getBetterRef(x_6, x_8); +lean_dec(x_6); +x_10 = l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1(x_1, x_2, x_3, x_7); +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) { -lean_object* x_9; -x_9 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_4); -lean_dec(x_1); -return x_9; -} +lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_12 = lean_ctor_get(x_10, 0); +x_13 = lean_ctor_get(x_10, 1); +x_14 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_12, x_8, x_2, x_3, x_13); +lean_dec(x_2); +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 0) +{ +lean_object* x_16; +x_16 = lean_ctor_get(x_14, 0); +lean_ctor_set(x_10, 1, x_16); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set_tag(x_14, 1); +lean_ctor_set(x_14, 0, x_10); +return x_14; } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___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 { -size_t x_9; size_t x_10; lean_object* x_11; -x_9 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_10 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_11 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1(x_1, x_2, x_9, x_10, x_5, x_6, x_7, x_8); -lean_dec(x_2); -return x_11; +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_14, 0); +x_18 = lean_ctor_get(x_14, 1); +lean_inc(x_18); +lean_inc(x_17); +lean_dec(x_14); +lean_ctor_set(x_10, 1, x_17); +lean_ctor_set(x_10, 0, x_9); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_10); +lean_ctor_set(x_19, 1, x_18); +return x_19; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__2___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; lean_object* x_7; -x_5 = lean_unbox_usize(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; +x_20 = lean_ctor_get(x_10, 0); +x_21 = lean_ctor_get(x_10, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_10); +x_22 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_20, x_8, x_2, x_3, x_21); lean_dec(x_2); -x_6 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_7 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__2(x_1, x_5, x_6, x_4); -return x_7; +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +if (lean_is_exclusive(x_22)) { + lean_ctor_release(x_22, 0); + lean_ctor_release(x_22, 1); + x_25 = x_22; +} else { + lean_dec_ref(x_22); + x_25 = lean_box(0); } +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_9); +lean_ctor_set(x_26, 1, x_23); +if (lean_is_scalar(x_25)) { + x_27 = lean_alloc_ctor(1, 2, 0); +} else { + x_27 = x_25; + lean_ctor_set_tag(x_27, 1); } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___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) { -_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_dec(x_3); -x_10 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__3(x_1, x_8, x_9, x_4, x_5, x_6, x_7); -lean_dec(x_1); -return x_10; +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_24); +return x_27; } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +} +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabMutualInductive___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -size_t x_4; size_t x_5; uint8_t x_6; lean_object* x_7; -x_4 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_5 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_6 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__4(x_1, x_4, x_5); -lean_dec(x_1); -x_7 = lean_box(x_6); -return x_7; -} +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; +x_6 = l_Lean_Elab_Command_getRef(x_3, x_4, x_5); +x_7 = lean_ctor_get(x_6, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_6, 1); +lean_inc(x_8); +lean_dec(x_6); +x_9 = l_Lean_replaceRef(x_1, x_7); +lean_dec(x_7); +x_10 = !lean_is_exclusive(x_3); +if (x_10 == 0) +{ +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_elabMutualInductive___spec__10(x_2, x_3, x_4, x_8); +return x_12; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___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: +else { -lean_object* x_9; -x_9 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; lean_object* x_24; +x_13 = lean_ctor_get(x_3, 0); +x_14 = lean_ctor_get(x_3, 1); +x_15 = lean_ctor_get(x_3, 2); +x_16 = lean_ctor_get(x_3, 3); +x_17 = lean_ctor_get(x_3, 4); +x_18 = lean_ctor_get(x_3, 5); +x_19 = lean_ctor_get(x_3, 7); +x_20 = lean_ctor_get(x_3, 8); +x_21 = lean_ctor_get(x_3, 9); +x_22 = lean_ctor_get_uint8(x_3, sizeof(void*)*10); +lean_inc(x_21); +lean_inc(x_20); +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); lean_dec(x_3); -lean_dec(x_2); -return x_9; -} +x_23 = lean_alloc_ctor(0, 10, 1); +lean_ctor_set(x_23, 0, x_13); +lean_ctor_set(x_23, 1, x_14); +lean_ctor_set(x_23, 2, x_15); +lean_ctor_set(x_23, 3, x_16); +lean_ctor_set(x_23, 4, x_17); +lean_ctor_set(x_23, 5, x_18); +lean_ctor_set(x_23, 6, x_9); +lean_ctor_set(x_23, 7, x_19); +lean_ctor_set(x_23, 8, x_20); +lean_ctor_set(x_23, 9, x_21); +lean_ctor_set_uint8(x_23, sizeof(void*)*10, x_22); +x_24 = l_Lean_throwError___at_Lean_Elab_Command_elabMutualInductive___spec__10(x_2, x_23, x_4, x_8); +return x_24; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___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___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_2); -lean_dec(x_1); -return x_6; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___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_elabMutualInductive___spec__13(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_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields(x_1, x_2, x_3, x_4); -lean_dec(x_1); -return x_5; -} -} -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInductiveViews___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: +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_5 = l_Lean_Elab_Command_getRef(x_2, x_3, x_4); +x_6 = lean_ctor_get(x_5, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_5, 1); +lean_inc(x_7); +lean_dec(x_5); +x_8 = lean_ctor_get(x_2, 4); +lean_inc(x_8); +lean_inc(x_8); +x_9 = l_Lean_Elab_getBetterRef(x_6, x_8); +lean_dec(x_6); +x_10 = l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1(x_1, x_2, x_3, x_7); +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) { -uint8_t x_12; -x_12 = lean_usize_dec_lt(x_3, x_2); -if (x_12 == 0) +lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_12 = lean_ctor_get(x_10, 0); +x_13 = lean_ctor_get(x_10, 1); +x_14 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_12, x_8, x_2, x_3, x_13); +lean_dec(x_2); +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 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; +lean_object* x_16; +x_16 = lean_ctor_get(x_14, 0); +lean_ctor_set(x_10, 1, x_16); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set_tag(x_14, 1); +lean_ctor_set(x_14, 0, x_10); +return x_14; } else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; -lean_dec(x_4); -x_14 = lean_array_uget(x_1, x_3); -x_15 = lean_ctor_get(x_14, 4); -lean_inc(x_15); -lean_dec(x_14); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -x_16 = l_Lean_Meta_mkInjectiveTheorems(x_15, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_16) == 0) -{ -lean_object* x_17; size_t x_18; size_t x_19; lean_object* x_20; -x_17 = lean_ctor_get(x_16, 1); +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_14, 0); +x_18 = lean_ctor_get(x_14, 1); +lean_inc(x_18); lean_inc(x_17); -lean_dec(x_16); -x_18 = 1; -x_19 = lean_usize_add(x_3, x_18); -x_20 = lean_box(0); -x_3 = x_19; -x_4 = x_20; -x_11 = x_17; -goto _start; +lean_dec(x_14); +lean_ctor_set(x_10, 1, x_17); +lean_ctor_set(x_10, 0, x_9); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_10); +lean_ctor_set(x_19, 1, x_18); +return x_19; } -else -{ -uint8_t x_22; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -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_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_20 = lean_ctor_get(x_10, 0); +x_21 = lean_ctor_get(x_10, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_10); +x_22 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_20, x_8, x_2, x_3, x_21); +lean_dec(x_2); +x_23 = lean_ctor_get(x_22, 0); 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; +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +if (lean_is_exclusive(x_22)) { + lean_ctor_release(x_22, 0); + lean_ctor_release(x_22, 1); + x_25 = x_22; +} else { + lean_dec_ref(x_22); + x_25 = lean_box(0); } +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_9); +lean_ctor_set(x_26, 1, x_23); +if (lean_is_scalar(x_25)) { + x_27 = lean_alloc_ctor(1, 2, 0); +} else { + x_27 = x_25; + lean_ctor_set_tag(x_27, 1); } +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_24); +return x_27; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInductiveViews___spec__2(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_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_Command_elabMutualInductive___spec__12(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _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_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; +x_6 = l_Lean_Elab_Command_getRef(x_3, x_4, x_5); +x_7 = lean_ctor_get(x_6, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_6, 1); +lean_inc(x_8); lean_dec(x_6); -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; +x_9 = l_Lean_replaceRef(x_1, x_7); +lean_dec(x_7); +x_10 = !lean_is_exclusive(x_3); +if (x_10 == 0) +{ +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_elabMutualInductive___spec__13(x_2, x_3, x_4, x_8); +return x_12; } else { -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_dec(x_4); -x_14 = lean_array_uget(x_1, x_3); -x_15 = lean_ctor_get(x_14, 4); -lean_inc(x_15); -x_16 = lean_ctor_get(x_14, 2); -lean_inc(x_16); -lean_dec(x_14); -x_17 = lean_ctor_get(x_16, 1); -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); -if (lean_obj_tag(x_19) == 0) -{ -lean_object* x_20; size_t x_21; size_t x_22; lean_object* x_23; -x_20 = lean_ctor_get(x_19, 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; uint8_t x_22; lean_object* x_23; lean_object* x_24; +x_13 = lean_ctor_get(x_3, 0); +x_14 = lean_ctor_get(x_3, 1); +x_15 = lean_ctor_get(x_3, 2); +x_16 = lean_ctor_get(x_3, 3); +x_17 = lean_ctor_get(x_3, 4); +x_18 = lean_ctor_get(x_3, 5); +x_19 = lean_ctor_get(x_3, 7); +x_20 = lean_ctor_get(x_3, 8); +x_21 = lean_ctor_get(x_3, 9); +x_22 = lean_ctor_get_uint8(x_3, sizeof(void*)*10); +lean_inc(x_21); lean_inc(x_20); -lean_dec(x_19); -x_21 = 1; -x_22 = lean_usize_add(x_3, x_21); -x_23 = lean_box(0); -x_3 = x_22; -x_4 = x_23; -x_11 = x_20; -goto _start; +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_dec(x_3); +x_23 = lean_alloc_ctor(0, 10, 1); +lean_ctor_set(x_23, 0, x_13); +lean_ctor_set(x_23, 1, x_14); +lean_ctor_set(x_23, 2, x_15); +lean_ctor_set(x_23, 3, x_16); +lean_ctor_set(x_23, 4, x_17); +lean_ctor_set(x_23, 5, x_18); +lean_ctor_set(x_23, 6, x_9); +lean_ctor_set(x_23, 7, x_19); +lean_ctor_set(x_23, 8, x_20); +lean_ctor_set(x_23, 9, x_21); +lean_ctor_set_uint8(x_23, sizeof(void*)*10, x_22); +x_24 = l_Lean_throwError___at_Lean_Elab_Command_elabMutualInductive___spec__13(x_2, x_23, x_4, x_8); +return x_24; } -else +} +} +LEAN_EXPORT lean_object* l_Lean_getDocStringText___at_Lean_Elab_Command_elabMutualInductive___spec__11(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: { -uint8_t x_25; -lean_dec(x_10); +lean_object* x_5; lean_object* x_6; +x_5 = lean_unsigned_to_nat(1u); +x_6 = l_Lean_Syntax_getArg(x_1, x_5); +if (lean_obj_tag(x_6) == 2) +{ +uint8_t x_7; +lean_dec(x_2); +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; +x_8 = lean_ctor_get(x_6, 1); +x_9 = lean_ctor_get(x_6, 0); lean_dec(x_9); +x_10 = lean_string_utf8_byte_size(x_8); +x_11 = lean_unsigned_to_nat(2u); +x_12 = lean_nat_sub(x_10, x_11); +lean_dec(x_10); +x_13 = lean_unsigned_to_nat(0u); +x_14 = lean_string_utf8_extract(x_8, x_13, x_12); +lean_dec(x_12); 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) +lean_ctor_set_tag(x_6, 0); +lean_ctor_set(x_6, 1, x_4); +lean_ctor_set(x_6, 0, x_14); +return x_6; +} +else { -return x_19; +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_15 = lean_ctor_get(x_6, 1); +lean_inc(x_15); +lean_dec(x_6); +x_16 = lean_string_utf8_byte_size(x_15); +x_17 = lean_unsigned_to_nat(2u); +x_18 = lean_nat_sub(x_16, x_17); +lean_dec(x_16); +x_19 = lean_unsigned_to_nat(0u); +x_20 = lean_string_utf8_extract(x_15, x_19, x_18); +lean_dec(x_18); +lean_dec(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_4); +return x_21; +} } 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_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); +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 = l_Lean_MessageData_ofSyntax(x_6); +x_23 = l_Lean_indentD(x_22); +x_24 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__2; +x_25 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_25, 0, x_24); +lean_ctor_set(x_25, 1, x_23); +x_26 = l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3; +x_27 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +x_28 = l_Lean_throwErrorAt___at_Lean_Elab_Command_elabMutualInductive___spec__12(x_1, x_27, x_2, x_3, x_4); return x_28; } } } -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInductiveViews___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_elabModifiers___at_Lean_Elab_Command_elabMutualInductive___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -uint8_t x_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); -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); -x_15 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl(x_2, x_3, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_15) == 0) -{ -lean_object* x_16; lean_object* x_17; -x_16 = lean_ctor_get(x_15, 1); -lean_inc(x_16); -lean_dec(x_15); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_4); -x_17 = l_Lean_Meta_mkSizeOfInstances(x_4, x_7, x_8, x_9, x_10, x_16); -if (lean_obj_tag(x_17) == 0) -{ -lean_object* x_18; lean_object* x_19; -x_18 = lean_ctor_get(x_17, 1); -lean_inc(x_18); -lean_dec(x_17); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -x_19 = l_Lean_Meta_IndPredBelow_mkBelow(x_4, x_7, x_8, x_9, x_10, x_18); -if (lean_obj_tag(x_19) == 0) -{ -lean_object* x_20; size_t x_21; size_t x_22; lean_object* x_23; lean_object* x_24; -x_20 = lean_ctor_get(x_19, 1); -lean_inc(x_20); -lean_dec(x_19); -x_21 = lean_array_size(x_3); -x_22 = 0; -x_23 = lean_box(0); -x_24 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInductiveViews___spec__1(x_3, x_21, x_22, x_23, x_5, x_6, x_7, x_8, x_9, x_10, x_20); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -if (lean_obj_tag(x_24) == 0) +uint8_t x_11; uint8_t x_12; +x_11 = l_Lean_Syntax_isNone(x_1); +x_12 = l_Lean_Syntax_isNone(x_2); +if (x_11 == 0) { -uint8_t x_25; -x_25 = !lean_is_exclusive(x_24); -if (x_25 == 0) +if (x_12 == 0) { -lean_object* x_26; -x_26 = lean_ctor_get(x_24, 0); -lean_dec(x_26); -lean_ctor_set(x_24, 0, x_23); -return x_24; +uint8_t x_13; lean_object* x_14; lean_object* x_15; +x_13 = 1; +x_14 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_14, 0, x_3); +lean_ctor_set(x_14, 1, x_4); +lean_ctor_set(x_14, 2, x_7); +lean_ctor_set_uint8(x_14, sizeof(void*)*3, x_5); +lean_ctor_set_uint8(x_14, sizeof(void*)*3 + 1, x_13); +lean_ctor_set_uint8(x_14, sizeof(void*)*3 + 2, x_6); +lean_ctor_set_uint8(x_14, sizeof(void*)*3 + 3, x_13); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_10); +return x_15; } else { -lean_object* x_27; lean_object* x_28; -x_27 = lean_ctor_get(x_24, 1); -lean_inc(x_27); -lean_dec(x_24); -x_28 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_28, 0, x_23); -lean_ctor_set(x_28, 1, x_27); -return x_28; +uint8_t x_16; uint8_t x_17; lean_object* x_18; lean_object* x_19; +x_16 = 1; +x_17 = 0; +x_18 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_18, 0, x_3); +lean_ctor_set(x_18, 1, x_4); +lean_ctor_set(x_18, 2, x_7); +lean_ctor_set_uint8(x_18, sizeof(void*)*3, x_5); +lean_ctor_set_uint8(x_18, sizeof(void*)*3 + 1, x_16); +lean_ctor_set_uint8(x_18, sizeof(void*)*3 + 2, x_6); +lean_ctor_set_uint8(x_18, sizeof(void*)*3 + 3, x_17); +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set(x_19, 1, x_10); +return x_19; } } else { -uint8_t x_29; -x_29 = !lean_is_exclusive(x_24); -if (x_29 == 0) +if (x_12 == 0) { -return x_24; +uint8_t x_20; uint8_t x_21; lean_object* x_22; lean_object* x_23; +x_20 = 0; +x_21 = 1; +x_22 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_22, 0, x_3); +lean_ctor_set(x_22, 1, x_4); +lean_ctor_set(x_22, 2, x_7); +lean_ctor_set_uint8(x_22, sizeof(void*)*3, x_5); +lean_ctor_set_uint8(x_22, sizeof(void*)*3 + 1, x_20); +lean_ctor_set_uint8(x_22, sizeof(void*)*3 + 2, x_6); +lean_ctor_set_uint8(x_22, sizeof(void*)*3 + 3, x_21); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_10); +return x_23; } else { -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; +uint8_t x_24; lean_object* x_25; lean_object* x_26; +x_24 = 0; +x_25 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_25, 0, x_3); +lean_ctor_set(x_25, 1, x_4); +lean_ctor_set(x_25, 2, x_7); +lean_ctor_set_uint8(x_25, sizeof(void*)*3, x_5); +lean_ctor_set_uint8(x_25, sizeof(void*)*3 + 1, x_24); +lean_ctor_set_uint8(x_25, sizeof(void*)*3 + 2, x_6); +lean_ctor_set_uint8(x_25, sizeof(void*)*3 + 3, x_24); +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_10); +return x_26; } } } -else +} +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualInductive___spec__1___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, lean_object* x_6, uint8_t x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: { -uint8_t x_33; -lean_dec(x_9); -lean_dec(x_10); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -x_33 = !lean_is_exclusive(x_19); -if (x_33 == 0) +lean_object* x_11; +x_11 = l_Lean_Syntax_getOptional_x3f(x_6); +if (lean_obj_tag(x_11) == 0) { -return x_19; +lean_object* x_12; lean_object* x_13; +x_12 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__8___closed__1; +x_13 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualInductive___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_7, x_5, x_12, x_8, x_9, x_10); +lean_dec(x_8); +return x_13; } else { -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_19, 0); -x_35 = lean_ctor_get(x_19, 1); -lean_inc(x_35); -lean_inc(x_34); -lean_dec(x_19); -x_36 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_36, 0, x_34); -lean_ctor_set(x_36, 1, x_35); -return x_36; -} -} +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_11, 0); +lean_inc(x_14); +lean_dec(x_11); +lean_inc(x_8); +x_15 = l_Lean_Elab_elabDeclAttrs___at_Lean_Elab_Command_elabMutualInductive___spec__2(x_14, x_8, x_9, x_10); +lean_dec(x_14); +if (lean_obj_tag(x_15) == 0) +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_15, 1); +lean_inc(x_17); +lean_dec(x_15); +x_18 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualInductive___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_7, x_5, x_16, x_8, x_9, x_17); +lean_dec(x_8); +return x_18; } else { -uint8_t x_37; -lean_dec(x_9); -lean_dec(x_10); +uint8_t x_19; lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_37 = !lean_is_exclusive(x_17); -if (x_37 == 0) +x_19 = !lean_is_exclusive(x_15); +if (x_19 == 0) { -return x_17; +return x_15; } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_17, 0); -x_39 = lean_ctor_get(x_17, 1); -lean_inc(x_39); -lean_inc(x_38); -lean_dec(x_17); -x_40 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_40, 0, x_38); -lean_ctor_set(x_40, 1, x_39); -return x_40; +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_15, 0); +x_21 = lean_ctor_get(x_15, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_15); +x_22 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_22, 0, x_20); +lean_ctor_set(x_22, 1, x_21); +return x_22; +} } } } +} +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualInductive___spec__1___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_Syntax_getOptional_x3f(x_6); +if (lean_obj_tag(x_11) == 0) +{ +uint8_t x_12; lean_object* x_13; +x_12 = 0; +x_13 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualInductive___spec__1___lambda__2(x_1, x_2, x_3, x_7, x_4, x_5, x_12, x_8, x_9, x_10); +return x_13; +} else { -uint8_t x_41; -lean_dec(x_9); -lean_dec(x_10); -lean_dec(x_8); +lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_14 = lean_ctor_get(x_11, 0); +lean_inc(x_14); +lean_dec(x_11); +lean_inc(x_14); +x_15 = l_Lean_Syntax_getKind(x_14); +x_16 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__2; +x_17 = lean_name_eq(x_15, x_16); +if (x_17 == 0) +{ +lean_object* x_18; uint8_t x_19; +x_18 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__4; +x_19 = lean_name_eq(x_15, x_18); +lean_dec(x_15); +if (x_19 == 0) +{ +lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); lean_dec(x_3); -x_41 = !lean_is_exclusive(x_15); -if (x_41 == 0) +x_20 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__6; +x_21 = l_Lean_throwErrorAt___at_Lean_Elab_Command_elabMutualInductive___spec__9(x_14, x_20, x_8, x_9, x_10); +lean_dec(x_14); +x_22 = !lean_is_exclusive(x_21); +if (x_22 == 0) { -return x_15; +return x_21; } else { -lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_ctor_get(x_15, 0); -x_43 = lean_ctor_get(x_15, 1); -lean_inc(x_43); -lean_inc(x_42); -lean_dec(x_15); -x_44 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_44, 0, x_42); -lean_ctor_set(x_44, 1, x_43); -return x_44; -} +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_21, 0); +x_24 = lean_ctor_get(x_21, 1); +lean_inc(x_24); +lean_inc(x_23); +lean_dec(x_21); +x_25 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +return x_25; } } else { -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; uint8_t x_56; lean_object* x_57; uint8_t x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; -x_45 = lean_ctor_get(x_9, 0); -x_46 = lean_ctor_get(x_9, 1); -x_47 = lean_ctor_get(x_9, 2); -x_48 = lean_ctor_get(x_9, 3); -x_49 = lean_ctor_get(x_9, 4); -x_50 = lean_ctor_get(x_9, 5); -x_51 = lean_ctor_get(x_9, 6); -x_52 = lean_ctor_get(x_9, 7); -x_53 = lean_ctor_get(x_9, 8); -x_54 = lean_ctor_get(x_9, 9); -x_55 = lean_ctor_get(x_9, 10); -x_56 = lean_ctor_get_uint8(x_9, sizeof(void*)*12); -x_57 = lean_ctor_get(x_9, 11); -x_58 = lean_ctor_get_uint8(x_9, sizeof(void*)*12 + 1); -lean_inc(x_57); -lean_inc(x_55); -lean_inc(x_54); -lean_inc(x_53); -lean_inc(x_52); -lean_inc(x_51); -lean_inc(x_50); -lean_inc(x_49); -lean_inc(x_48); -lean_inc(x_47); -lean_inc(x_46); -lean_inc(x_45); -lean_dec(x_9); -x_59 = l_Lean_replaceRef(x_1, x_50); -lean_dec(x_50); -x_60 = lean_alloc_ctor(0, 12, 2); -lean_ctor_set(x_60, 0, x_45); -lean_ctor_set(x_60, 1, x_46); -lean_ctor_set(x_60, 2, x_47); -lean_ctor_set(x_60, 3, x_48); -lean_ctor_set(x_60, 4, x_49); -lean_ctor_set(x_60, 5, x_59); -lean_ctor_set(x_60, 6, x_51); -lean_ctor_set(x_60, 7, x_52); -lean_ctor_set(x_60, 8, x_53); -lean_ctor_set(x_60, 9, x_54); -lean_ctor_set(x_60, 10, x_55); -lean_ctor_set(x_60, 11, x_57); -lean_ctor_set_uint8(x_60, sizeof(void*)*12, x_56); -lean_ctor_set_uint8(x_60, sizeof(void*)*12 + 1, x_58); -lean_inc(x_10); -lean_inc(x_60); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_3); -x_61 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl(x_2, x_3, x_5, x_6, x_7, x_8, x_60, x_10, x_11); -if (lean_obj_tag(x_61) == 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); -lean_inc(x_10); -lean_inc(x_60); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_4); -x_63 = l_Lean_Meta_mkSizeOfInstances(x_4, x_7, x_8, x_60, x_10, x_62); -if (lean_obj_tag(x_63) == 0) +uint8_t x_26; lean_object* x_27; +lean_dec(x_14); +x_26 = 1; +x_27 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualInductive___spec__1___lambda__2(x_1, x_2, x_3, x_7, x_4, x_5, x_26, x_8, x_9, x_10); +return x_27; +} +} +else { -lean_object* x_64; lean_object* x_65; -x_64 = lean_ctor_get(x_63, 1); -lean_inc(x_64); -lean_dec(x_63); -lean_inc(x_10); -lean_inc(x_60); -lean_inc(x_8); -lean_inc(x_7); -x_65 = l_Lean_Meta_IndPredBelow_mkBelow(x_4, x_7, x_8, x_60, x_10, x_64); -if (lean_obj_tag(x_65) == 0) +uint8_t x_28; lean_object* x_29; +lean_dec(x_15); +lean_dec(x_14); +x_28 = 2; +x_29 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualInductive___spec__1___lambda__2(x_1, x_2, x_3, x_7, x_4, x_5, x_28, x_8, x_9, x_10); +return x_29; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualInductive___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: { -lean_object* x_66; size_t x_67; size_t x_68; lean_object* x_69; lean_object* x_70; -x_66 = lean_ctor_get(x_65, 1); -lean_inc(x_66); -lean_dec(x_65); -x_67 = lean_array_size(x_3); -x_68 = 0; -x_69 = lean_box(0); -x_70 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInductiveViews___spec__1(x_3, x_67, x_68, x_69, x_5, x_6, x_7, x_8, x_60, x_10, x_66); +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; uint8_t x_19; +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Lean_Syntax_getArg(x_1, x_5); +x_7 = lean_unsigned_to_nat(1u); +x_8 = l_Lean_Syntax_getArg(x_1, x_7); +x_9 = lean_unsigned_to_nat(2u); +x_10 = l_Lean_Syntax_getArg(x_1, x_9); +x_11 = lean_unsigned_to_nat(3u); +x_12 = l_Lean_Syntax_getArg(x_1, x_11); +x_13 = lean_unsigned_to_nat(4u); +x_14 = l_Lean_Syntax_getArg(x_1, x_13); +x_15 = lean_unsigned_to_nat(5u); +x_16 = l_Lean_Syntax_getArg(x_1, x_15); +x_17 = l_Lean_Syntax_isNone(x_16); +x_18 = l_Lean_Syntax_getOptional_x3f(x_6); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -if (lean_obj_tag(x_70) == 0) +if (x_17 == 0) { -lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_71 = lean_ctor_get(x_70, 1); -lean_inc(x_71); -if (lean_is_exclusive(x_70)) { - lean_ctor_release(x_70, 0); - lean_ctor_release(x_70, 1); - x_72 = x_70; -} else { - lean_dec_ref(x_70); - x_72 = lean_box(0); -} -if (lean_is_scalar(x_72)) { - x_73 = lean_alloc_ctor(0, 2, 0); -} else { - x_73 = x_72; -} -lean_ctor_set(x_73, 0, x_69); -lean_ctor_set(x_73, 1, x_71); -return x_73; +lean_object* x_43; lean_object* x_44; lean_object* x_45; uint8_t x_46; +x_43 = l_Lean_Syntax_getArg(x_16, x_5); +lean_dec(x_16); +x_44 = l_Lean_Syntax_getKind(x_43); +x_45 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__2; +x_46 = lean_name_eq(x_44, x_45); +lean_dec(x_44); +if (x_46 == 0) +{ +uint8_t x_47; +x_47 = 1; +x_19 = x_47; +goto block_42; } else { -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); -x_75 = lean_ctor_get(x_70, 1); -lean_inc(x_75); -if (lean_is_exclusive(x_70)) { - lean_ctor_release(x_70, 0); - lean_ctor_release(x_70, 1); - x_76 = x_70; -} else { - lean_dec_ref(x_70); - x_76 = lean_box(0); +uint8_t x_48; +x_48 = 0; +x_19 = x_48; +goto block_42; } -if (lean_is_scalar(x_76)) { - x_77 = lean_alloc_ctor(1, 2, 0); -} else { - x_77 = x_76; } -lean_ctor_set(x_77, 0, x_74); -lean_ctor_set(x_77, 1, x_75); -return x_77; +else +{ +uint8_t x_49; +lean_dec(x_16); +x_49 = 2; +x_19 = x_49; +goto block_42; } +block_42: +{ +if (lean_obj_tag(x_18) == 0) +{ +lean_object* x_20; lean_object* x_21; +x_20 = lean_box(0); +x_21 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualInductive___spec__1___lambda__3(x_12, x_14, x_1, x_19, x_8, x_10, x_20, x_2, x_3, x_4); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_14); +lean_dec(x_12); +return x_21; } else { -lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; -lean_dec(x_60); +uint8_t x_22; +x_22 = !lean_is_exclusive(x_18); +if (x_22 == 0) +{ +lean_object* x_23; lean_object* x_24; +x_23 = lean_ctor_get(x_18, 0); +lean_inc(x_2); +x_24 = l_Lean_getDocStringText___at_Lean_Elab_Command_elabMutualInductive___spec__11(x_23, x_2, x_3, x_4); +lean_dec(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_24, 0); +lean_inc(x_25); +x_26 = lean_ctor_get(x_24, 1); +lean_inc(x_26); +lean_dec(x_24); +lean_ctor_set(x_18, 0, x_25); +x_27 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualInductive___spec__1___lambda__3(x_12, x_14, x_1, x_19, x_8, x_10, x_18, x_2, x_3, x_26); lean_dec(x_10); lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -x_78 = lean_ctor_get(x_65, 0); -lean_inc(x_78); -x_79 = lean_ctor_get(x_65, 1); -lean_inc(x_79); -if (lean_is_exclusive(x_65)) { - lean_ctor_release(x_65, 0); - lean_ctor_release(x_65, 1); - x_80 = x_65; -} else { - lean_dec_ref(x_65); - x_80 = lean_box(0); -} -if (lean_is_scalar(x_80)) { - x_81 = lean_alloc_ctor(1, 2, 0); -} else { - x_81 = x_80; -} -lean_ctor_set(x_81, 0, x_78); -lean_ctor_set(x_81, 1, x_79); -return x_81; -} +lean_dec(x_14); +lean_dec(x_12); +return x_27; } else { -lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; -lean_dec(x_60); +uint8_t x_28; +lean_free_object(x_18); +lean_dec(x_14); +lean_dec(x_12); 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); -x_82 = lean_ctor_get(x_63, 0); -lean_inc(x_82); -x_83 = lean_ctor_get(x_63, 1); -lean_inc(x_83); -if (lean_is_exclusive(x_63)) { - lean_ctor_release(x_63, 0); - lean_ctor_release(x_63, 1); - x_84 = x_63; -} else { - lean_dec_ref(x_63); - x_84 = lean_box(0); +lean_dec(x_2); +lean_dec(x_1); +x_28 = !lean_is_exclusive(x_24); +if (x_28 == 0) +{ +return x_24; +} +else +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_24, 0); +x_30 = lean_ctor_get(x_24, 1); +lean_inc(x_30); +lean_inc(x_29); +lean_dec(x_24); +x_31 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_31, 0, x_29); +lean_ctor_set(x_31, 1, x_30); +return x_31; } -if (lean_is_scalar(x_84)) { - x_85 = lean_alloc_ctor(1, 2, 0); -} else { - x_85 = x_84; } -lean_ctor_set(x_85, 0, x_82); -lean_ctor_set(x_85, 1, x_83); -return x_85; } +else +{ +lean_object* x_32; lean_object* x_33; +x_32 = lean_ctor_get(x_18, 0); +lean_inc(x_32); +lean_dec(x_18); +lean_inc(x_2); +x_33 = l_Lean_getDocStringText___at_Lean_Elab_Command_elabMutualInductive___spec__11(x_32, x_2, x_3, x_4); +lean_dec(x_32); +if (lean_obj_tag(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_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_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualInductive___spec__1___lambda__3(x_12, x_14, x_1, x_19, x_8, x_10, x_36, x_2, x_3, x_35); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_14); +lean_dec(x_12); +return x_37; } else { -lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; -lean_dec(x_60); +lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; +lean_dec(x_14); +lean_dec(x_12); 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); -x_86 = lean_ctor_get(x_61, 0); -lean_inc(x_86); -x_87 = lean_ctor_get(x_61, 1); -lean_inc(x_87); -if (lean_is_exclusive(x_61)) { - lean_ctor_release(x_61, 0); - lean_ctor_release(x_61, 1); - x_88 = x_61; +lean_dec(x_2); +lean_dec(x_1); +x_38 = lean_ctor_get(x_33, 0); +lean_inc(x_38); +x_39 = lean_ctor_get(x_33, 1); +lean_inc(x_39); +if (lean_is_exclusive(x_33)) { + lean_ctor_release(x_33, 0); + lean_ctor_release(x_33, 1); + x_40 = x_33; } else { - lean_dec_ref(x_61); - x_88 = lean_box(0); + lean_dec_ref(x_33); + x_40 = lean_box(0); } -if (lean_is_scalar(x_88)) { - x_89 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_40)) { + x_41 = lean_alloc_ctor(1, 2, 0); } else { - x_89 = x_88; + x_41 = x_40; } -lean_ctor_set(x_89, 0, x_86); -lean_ctor_set(x_89, 1, x_87); -return x_89; +lean_ctor_set(x_41, 0, x_38); +lean_ctor_set(x_41, 1, x_39); +return x_41; } } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInductiveViews___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_12 = lean_ctor_get(x_1, 4); -lean_inc(x_12); -lean_dec(x_1); -lean_inc(x_12); -x_13 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabInductiveViews___lambda__1___boxed), 11, 4); -lean_closure_set(x_13, 0, x_2); -lean_closure_set(x_13, 1, x_4); -lean_closure_set(x_13, 2, x_3); -lean_closure_set(x_13, 3, x_12); -x_14 = l_Lean_Elab_Term_withDeclName___rarg(x_12, x_13, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -return x_14; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInductiveViews___lambda__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_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabMutualInductive___spec__14(size_t x_1, size_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { -uint8_t x_12; -x_12 = !lean_is_exclusive(x_9); -if (x_12 == 0) -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -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 = 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); -if (lean_obj_tag(x_16) == 0) -{ -uint8_t x_17; -x_17 = !lean_is_exclusive(x_16); -if (x_17 == 0) +uint8_t x_7; +x_7 = lean_usize_dec_lt(x_2, x_1); +if (x_7 == 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; +lean_object* x_8; +lean_dec(x_4); +x_8 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_8, 0, x_3); +lean_ctor_set(x_8, 1, x_6); +return x_8; } 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; -} +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_3, x_2); +x_10 = lean_unsigned_to_nat(0u); +x_11 = lean_array_uset(x_3, x_2, x_10); +x_12 = l_Lean_Syntax_getArg(x_9, x_10); +lean_inc(x_4); +x_13 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualInductive___spec__1(x_12, x_4, x_5, x_6); +if (lean_obj_tag(x_13) == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; size_t x_19; size_t x_20; lean_object* x_21; +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_unsigned_to_nat(1u); +x_17 = l_Lean_Syntax_getArg(x_9, x_16); +lean_dec(x_9); +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_14); +lean_ctor_set(x_18, 1, x_17); +x_19 = 1; +x_20 = lean_usize_add(x_2, x_19); +x_21 = lean_array_uset(x_11, x_2, x_18); +x_2 = x_20; +x_3 = x_21; +x_6 = x_15; +goto _start; } else { -uint8_t x_21; -x_21 = !lean_is_exclusive(x_16); -if (x_21 == 0) +uint8_t x_23; +lean_dec(x_11); +lean_dec(x_9); +lean_dec(x_4); +x_23 = !lean_is_exclusive(x_13); +if (x_23 == 0) { -return x_16; +return x_13; } else { -lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_22 = lean_ctor_get(x_16, 0); -x_23 = lean_ctor_get(x_16, 1); -lean_inc(x_23); -lean_inc(x_22); -lean_dec(x_16); -x_24 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_24, 0, x_22); -lean_ctor_set(x_24, 1, x_23); -return x_24; +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_13, 0); +x_25 = lean_ctor_get(x_13, 1); +lean_inc(x_25); +lean_inc(x_24); +lean_dec(x_13); +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_EXPORT lean_object* l_Lean_Elab_Command_elabMutualInductive(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: { -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; lean_object* x_37; uint8_t x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_25 = lean_ctor_get(x_9, 0); -x_26 = lean_ctor_get(x_9, 1); -x_27 = lean_ctor_get(x_9, 2); -x_28 = lean_ctor_get(x_9, 3); -x_29 = lean_ctor_get(x_9, 4); -x_30 = lean_ctor_get(x_9, 5); -x_31 = lean_ctor_get(x_9, 6); -x_32 = lean_ctor_get(x_9, 7); -x_33 = lean_ctor_get(x_9, 8); -x_34 = lean_ctor_get(x_9, 9); -x_35 = lean_ctor_get(x_9, 10); -x_36 = lean_ctor_get_uint8(x_9, sizeof(void*)*12); -x_37 = lean_ctor_get(x_9, 11); -x_38 = lean_ctor_get_uint8(x_9, sizeof(void*)*12 + 1); -lean_inc(x_37); -lean_inc(x_35); -lean_inc(x_34); -lean_inc(x_33); -lean_inc(x_32); -lean_inc(x_31); -lean_inc(x_30); -lean_inc(x_29); -lean_inc(x_28); -lean_inc(x_27); -lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_9); -x_39 = l_Lean_replaceRef(x_1, x_30); -lean_dec(x_30); -x_40 = lean_alloc_ctor(0, 12, 2); -lean_ctor_set(x_40, 0, x_25); -lean_ctor_set(x_40, 1, x_26); -lean_ctor_set(x_40, 2, x_27); -lean_ctor_set(x_40, 3, x_28); -lean_ctor_set(x_40, 4, x_29); -lean_ctor_set(x_40, 5, x_39); -lean_ctor_set(x_40, 6, x_31); -lean_ctor_set(x_40, 7, x_32); -lean_ctor_set(x_40, 8, x_33); -lean_ctor_set(x_40, 9, x_34); -lean_ctor_set(x_40, 10, x_35); -lean_ctor_set(x_40, 11, x_37); -lean_ctor_set_uint8(x_40, sizeof(void*)*12, x_36); -lean_ctor_set_uint8(x_40, sizeof(void*)*12 + 1, x_38); -x_41 = lean_box(0); -x_42 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInductiveViews___spec__2(x_2, x_3, x_4, x_41, x_5, x_6, x_7, x_8, x_40, x_10, x_11); -if (lean_obj_tag(x_42) == 0) +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_array_size(x_1); +x_6 = 0; +lean_inc(x_2); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabMutualInductive___spec__14(x_5, x_6, x_1, x_2, x_3, x_4); +if (lean_obj_tag(x_7) == 0) { -lean_object* x_43; lean_object* x_44; lean_object* x_45; -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_42); - x_44 = lean_box(0); -} -if (lean_is_scalar(x_44)) { - x_45 = lean_alloc_ctor(0, 2, 0); -} else { - x_45 = x_44; +lean_object* x_8; lean_object* x_9; lean_object* x_10; +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_Elab_Command_elabInductives(x_8, x_2, x_3, x_9); +return x_10; } -lean_ctor_set(x_45, 0, x_41); -lean_ctor_set(x_45, 1, x_43); -return x_45; +else +{ +uint8_t x_11; +lean_dec(x_3); +lean_dec(x_2); +x_11 = !lean_is_exclusive(x_7); +if (x_11 == 0) +{ +return x_7; } 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); -lean_inc(x_46); -x_47 = lean_ctor_get(x_42, 1); -lean_inc(x_47); -if (lean_is_exclusive(x_42)) { - lean_ctor_release(x_42, 0); - lean_ctor_release(x_42, 1); - x_48 = x_42; -} else { - lean_dec_ref(x_42); - x_48 = lean_box(0); +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_7, 0); +x_13 = lean_ctor_get(x_7, 1); +lean_inc(x_13); +lean_inc(x_12); +lean_dec(x_7); +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; } -if (lean_is_scalar(x_48)) { - x_49 = lean_alloc_ctor(1, 2, 0); -} else { - x_49 = x_48; } -lean_ctor_set(x_49, 0, x_46); -lean_ctor_set(x_49, 1, x_47); -return x_49; } } +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabMutualInductive___spec__5___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_elabMutualInductive___spec__5(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; } } -static lean_object* _init_l_Lean_Elab_Command_elabInductiveViews___lambda__4___boxed__const__1() { +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabMutualInductive___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _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_5; +x_5 = l_Lean_throwError___at_Lean_Elab_Command_elabMutualInductive___spec__7(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInductiveViews___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabMutualInductive___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_12; size_t 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, 4); -lean_inc(x_12); +lean_object* x_6; +x_6 = l_Lean_throwErrorAt___at_Lean_Elab_Command_elabMutualInductive___spec__6(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_4); lean_dec(x_1); -x_13 = lean_array_size(x_2); -x_14 = lean_box_usize(x_13); -x_15 = l_Lean_Elab_Command_elabInductiveViews___lambda__4___boxed__const__1; -x_16 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabInductiveViews___lambda__3___boxed), 11, 4); -lean_closure_set(x_16, 0, x_3); -lean_closure_set(x_16, 1, x_2); -lean_closure_set(x_16, 2, x_14); -lean_closure_set(x_16, 3, x_15); -x_17 = l_Lean_Elab_Term_withDeclName___rarg(x_12, x_16, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -return x_17; +return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInductiveViews(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualInductive___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) { _start: { -lean_object* x_5; lean_object* x_29; lean_object* x_30; uint8_t x_31; -x_29 = lean_array_get_size(x_1); -x_30 = lean_unsigned_to_nat(0u); -x_31 = lean_nat_dec_lt(x_30, x_29); -lean_dec(x_29); -if (x_31 == 0) -{ -lean_object* x_32; lean_object* x_33; -x_32 = l_Lean_Elab_Command_instInhabitedInductiveView; -x_33 = l_outOfBounds___rarg(x_32); -x_5 = x_33; -goto block_28; +uint8_t x_7; lean_object* x_8; +x_7 = lean_unbox(x_1); +lean_dec(x_1); +x_8 = l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualInductive___spec__4___lambda__1(x_7, x_2, x_3, x_4, x_5, x_6); +lean_dec(x_5); +return x_8; } -else -{ -lean_object* x_34; -x_34 = lean_array_fget(x_1, x_30); -x_5 = x_34; -goto block_28; } -block_28: -{ -lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_6 = lean_ctor_get(x_5, 0); -lean_inc(x_6); -lean_inc(x_1); -lean_inc(x_6); -lean_inc(x_5); -x_7 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabInductiveViews___lambda__2), 11, 3); -lean_closure_set(x_7, 0, x_5); -lean_closure_set(x_7, 1, x_6); -lean_closure_set(x_7, 2, x_1); -x_8 = l_Lean_Elab_Command_runTermElabM___rarg(x_7, x_2, x_3, x_4); -if (lean_obj_tag(x_8) == 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_inc(x_3); -lean_inc(x_2); -x_10 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields(x_1, x_2, x_3, 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); -lean_inc(x_3); -lean_inc(x_2); -x_12 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers(x_1, x_2, x_3, x_11); -if (lean_obj_tag(x_12) == 0) +LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualInductive___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: { -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_ctor_get(x_12, 1); -lean_inc(x_13); -lean_dec(x_12); -x_14 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabInductiveViews___lambda__4___boxed), 11, 3); -lean_closure_set(x_14, 0, x_5); -lean_closure_set(x_14, 1, x_1); -lean_closure_set(x_14, 2, x_6); -x_15 = l_Lean_Elab_Command_runTermElabM___rarg(x_14, x_2, x_3, x_13); +lean_object* x_5; +x_5 = l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualInductive___spec__4(x_1, x_2, x_3, x_4); lean_dec(x_3); -lean_dec(x_2); -return x_15; +lean_dec(x_1); +return x_5; } -else +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabMutualInductive___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) { +_start: { -uint8_t x_16; -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); +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_dec(x_3); +x_10 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabMutualInductive___spec__8(x_1, x_8, x_9, x_4, x_5, x_6, x_7); +lean_dec(x_6); lean_dec(x_1); -x_16 = !lean_is_exclusive(x_12); -if (x_16 == 0) -{ -return x_12; +return x_10; } -else -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_12, 0); -x_18 = lean_ctor_get(x_12, 1); -lean_inc(x_18); -lean_inc(x_17); -lean_dec(x_12); -x_19 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_19, 0, x_17); -lean_ctor_set(x_19, 1, x_18); -return x_19; } +LEAN_EXPORT lean_object* l_Lean_Elab_elabAttrs___at_Lean_Elab_Command_elabMutualInductive___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Lean_Elab_elabAttrs___at_Lean_Elab_Command_elabMutualInductive___spec__3(x_1, x_2, x_3, x_4); +lean_dec(x_3); +lean_dec(x_1); +return x_5; } } -else +LEAN_EXPORT lean_object* l_Lean_Elab_elabDeclAttrs___at_Lean_Elab_Command_elabMutualInductive___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: { -uint8_t x_20; -lean_dec(x_6); -lean_dec(x_5); +lean_object* x_5; +x_5 = l_Lean_Elab_elabDeclAttrs___at_Lean_Elab_Command_elabMutualInductive___spec__2(x_1, x_2, x_3, x_4); lean_dec(x_3); -lean_dec(x_2); lean_dec(x_1); -x_20 = !lean_is_exclusive(x_10); -if (x_20 == 0) -{ -return x_10; +return x_5; } -else -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_10, 0); -x_22 = lean_ctor_get(x_10, 1); -lean_inc(x_22); -lean_inc(x_21); -lean_dec(x_10); -x_23 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_23, 0, x_21); -lean_ctor_set(x_23, 1, x_22); -return x_23; } +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabMutualInductive___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_Lean_throwError___at_Lean_Elab_Command_elabMutualInductive___spec__10(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; } } -else +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabMutualInductive___spec__9___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_24; -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -lean_dec(x_2); +lean_object* x_6; +x_6 = l_Lean_throwErrorAt___at_Lean_Elab_Command_elabMutualInductive___spec__9(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_4); lean_dec(x_1); -x_24 = !lean_is_exclusive(x_8); -if (x_24 == 0) -{ -return x_8; +return x_6; } -else -{ -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_8, 0); -x_26 = lean_ctor_get(x_8, 1); -lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_8); -x_27 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_26); -return x_27; } +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabMutualInductive___spec__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_throwError___at_Lean_Elab_Command_elabMutualInductive___spec__13(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; } } +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabMutualInductive___spec__12___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; +x_6 = l_Lean_throwErrorAt___at_Lean_Elab_Command_elabMutualInductive___spec__12(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_4); +lean_dec(x_1); +return x_6; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInductiveViews___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_getDocStringText___at_Lean_Elab_Command_elabMutualInductive___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _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_object* x_5; +x_5 = l_Lean_getDocStringText___at_Lean_Elab_Command_elabMutualInductive___spec__11(x_1, x_2, x_3, x_4); lean_dec(x_3); -x_14 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInductiveViews___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; +return x_5; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInductiveViews___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualInductive___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -size_t x_12; size_t x_13; lean_object* x_14; -x_12 = lean_unbox_usize(x_2); +uint8_t x_11; uint8_t x_12; lean_object* x_13; +x_11 = lean_unbox(x_5); +lean_dec(x_5); +x_12 = lean_unbox(x_6); +lean_dec(x_6); +x_13 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualInductive___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_11, x_12, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_8); lean_dec(x_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_1); -return x_14; +return x_13; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInductiveViews___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_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_elabModifiers___at_Lean_Elab_Command_elabMutualInductive___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: { -lean_object* x_12; -x_12 = l_Lean_Elab_Command_elabInductiveViews___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +uint8_t x_11; uint8_t x_12; lean_object* x_13; +x_11 = lean_unbox(x_5); +lean_dec(x_5); +x_12 = lean_unbox(x_7); +lean_dec(x_7); +x_13 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualInductive___spec__1___lambda__2(x_1, x_2, x_3, x_4, x_11, x_6, x_12, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_2); lean_dec(x_1); -return x_12; +return x_13; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInductiveViews___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualInductive___spec__1___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -size_t x_12; size_t x_13; lean_object* x_14; -x_12 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_13 = lean_unbox_usize(x_4); +uint8_t x_11; lean_object* x_12; +x_11 = lean_unbox(x_4); lean_dec(x_4); -x_14 = l_Lean_Elab_Command_elabInductiveViews___lambda__3(x_1, x_2, x_12, x_13, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_12 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualInductive___spec__1___lambda__3(x_1, x_2, x_3, x_11, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_5); lean_dec(x_2); lean_dec(x_1); -return x_14; +return x_12; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInductiveViews___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualInductive___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_12; -x_12 = l_Lean_Elab_Command_elabInductiveViews___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_4); -return x_12; +lean_object* x_5; +x_5 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualInductive___spec__1(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabMutualInductive___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) { +_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_2); +lean_dec(x_2); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabMutualInductive___spec__14(x_7, x_8, x_3, x_4, x_5, x_6); +lean_dec(x_5); +return x_9; } } lean_object* initialize_Lean_Util_ForEachExprWhere(uint8_t builtin, lean_object*); @@ -36561,6 +45013,7 @@ lean_object* initialize_Lean_Elab_ComputedFields(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Elab_DefView(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Elab_DeclUtil(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Elab_Deriving_Basic(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Elab_DeclarationRange(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Lean_Elab_Inductive(uint8_t builtin, lean_object* w) { lean_object * res; @@ -36608,6 +45061,9 @@ lean_dec_ref(res); res = initialize_Lean_Elab_Deriving_Basic(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +res = initialize_Lean_Elab_DeclarationRange(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__1 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__1(); lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__1); l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__2 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_4____closed__2(); @@ -36719,8 +45175,128 @@ l_Lean_Elab_Command_instInhabitedElabHeaderResult___closed__8 = _init_l_Lean_Ela lean_mark_persistent(l_Lean_Elab_Command_instInhabitedElabHeaderResult___closed__8); l_Lean_Elab_Command_instInhabitedElabHeaderResult = _init_l_Lean_Elab_Command_instInhabitedElabHeaderResult(); lean_mark_persistent(l_Lean_Elab_Command_instInhabitedElabHeaderResult); -l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__3___closed__1 = _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__3___closed__1(); -lean_mark_persistent(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__3___closed__1); +l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__1 = _init_l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__1(); +lean_mark_persistent(l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__1); +l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__2 = _init_l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__2(); +lean_mark_persistent(l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__2); +l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__3 = _init_l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__3(); +lean_mark_persistent(l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__3); +l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__4 = _init_l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__4(); +lean_mark_persistent(l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__4); +l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__5 = _init_l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__5(); +lean_mark_persistent(l_Lean_addDeclarationRanges___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___closed__5); +l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__1 = _init_l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__1); +l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2 = _init_l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___lambda__1___closed__2); +l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__1 = _init_l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__1(); +lean_mark_persistent(l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__1); +l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__2 = _init_l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__2(); +lean_mark_persistent(l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__2); +l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__3 = _init_l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__3(); +lean_mark_persistent(l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___closed__3); +l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__1 = _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__1(); +lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__1); +l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__2 = _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__2(); +lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__2); +l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__3 = _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__3(); +lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__3); +l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__4 = _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__4(); +lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__4); +l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__5 = _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__5(); +lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__5); +l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__6 = _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__6(); +lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__13___closed__6); +l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__14___rarg___closed__1 = _init_l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__14___rarg___closed__1(); +lean_mark_persistent(l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__14___rarg___closed__1); +l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__14___rarg___closed__2 = _init_l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__14___rarg___closed__2(); +lean_mark_persistent(l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__14___rarg___closed__2); +l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__1___closed__1 = _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__1___closed__1); +l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__1___closed__2 = _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__1___closed__2); +l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__1___closed__3 = _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__1___closed__3); +l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__2___closed__1 = _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__2___closed__1); +l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__2___closed__2 = _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__2___closed__2(); +lean_mark_persistent(l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__2___closed__2); +l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__2___closed__3 = _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__2___closed__3(); +lean_mark_persistent(l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__2___closed__3); +l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__2___closed__4 = _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__2___closed__4(); +lean_mark_persistent(l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___lambda__2___closed__4); +l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__1 = _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__1(); +lean_mark_persistent(l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__1); +l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__2 = _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__2(); +lean_mark_persistent(l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__2); +l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__3 = _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__3(); +lean_mark_persistent(l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__3); +l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__4 = _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__4(); +lean_mark_persistent(l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__4); +l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__5 = _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__5(); +lean_mark_persistent(l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__5); +l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__6 = _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__6(); +lean_mark_persistent(l_Lean_Elab_elabAttr___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__9___closed__6); +l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__8___closed__1 = _init_l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__8___closed__1(); +lean_mark_persistent(l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__8___closed__1); +l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__1 = _init_l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__1(); +lean_mark_persistent(l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__1); +l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__2 = _init_l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__2(); +lean_mark_persistent(l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__2); +l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3 = _init_l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3(); +lean_mark_persistent(l_Lean_getDocStringText___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__19___closed__3); +l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__1 = _init_l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__1); +l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__2 = _init_l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__2(); +lean_mark_persistent(l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__2); +l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__3 = _init_l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__3(); +lean_mark_persistent(l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__3); +l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__4 = _init_l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__4(); +lean_mark_persistent(l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__4); +l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__5 = _init_l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__5(); +lean_mark_persistent(l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__5); +l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__6 = _init_l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__6(); +lean_mark_persistent(l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___lambda__3___closed__6); +l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__1 = _init_l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__1(); +lean_mark_persistent(l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__1); +l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__2 = _init_l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__2(); +lean_mark_persistent(l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__2); +l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__2___closed__1 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__2___closed__1(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__2___closed__1); +l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__2___closed__2 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__2___closed__2(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__2___closed__2); +l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__3___closed__1 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__3___closed__1(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__3___closed__1); +l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__3___closed__2 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__3___closed__2(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___lambda__3___closed__2); +l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___closed__1 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___closed__1(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___closed__1); +l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___closed__2 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___closed__2(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___closed__2); +l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___closed__3 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___closed__3(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__23___closed__3); +l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__1 = _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__1(); +lean_mark_persistent(l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__1); +l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__2 = _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__2(); +lean_mark_persistent(l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__2); +l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__3 = _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__3(); +lean_mark_persistent(l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__3); +l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__4 = _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__4(); +lean_mark_persistent(l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__4); +l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__5 = _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__5(); +lean_mark_persistent(l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__5); +l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__6 = _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__6(); +lean_mark_persistent(l_Lean_Linter_logLint___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__26___closed__6); +l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1 = _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1(); +lean_mark_persistent(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1); +l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___closed__2 = _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___closed__2(); +lean_mark_persistent(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___closed__2); +l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___closed__3 = _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___closed__3(); +lean_mark_persistent(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___closed__3); +l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___closed__4 = _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___closed__4(); +lean_mark_persistent(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___closed__4); +l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___closed__5 = _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___closed__5(); +lean_mark_persistent(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___closed__5); l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__4___closed__1 = _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__4___closed__1(); lean_mark_persistent(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__4___closed__1); l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__4___closed__2 = _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__4___closed__2(); @@ -36733,8 +45309,6 @@ l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6__ lean_mark_persistent(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__3); l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__4 = _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__4(); lean_mark_persistent(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__4); -l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5 = _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5(); -lean_mark_persistent(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__5); l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams___spec__1___closed__1 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams___spec__1___closed__1(); lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams___spec__1___closed__1); l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams___spec__1___closed__2 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams___spec__1___closed__2(); @@ -36743,10 +45317,10 @@ l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe___spec__1___closed__1); l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe___spec__1___closed__2 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe___spec__1___closed__2(); lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe___spec__1___closed__2); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkLevelNames___spec__1___closed__1 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkLevelNames___spec__1___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkLevelNames___spec__1___closed__1); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkLevelNames___spec__1___closed__2 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkLevelNames___spec__1___closed__2(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkLevelNames___spec__1___closed__2); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_InductiveView_checkLevelNames___spec__1___closed__1 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_InductiveView_checkLevelNames___spec__1___closed__1(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_InductiveView_checkLevelNames___spec__1___closed__1); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_InductiveView_checkLevelNames___spec__1___closed__2 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_InductiveView_checkLevelNames___spec__1___closed__2(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_InductiveView_checkLevelNames___spec__1___closed__2); l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___rarg___closed__1 = _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___rarg___closed__1(); lean_mark_persistent(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___rarg___closed__1); l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___rarg___closed__2 = _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___rarg___closed__2(); @@ -36899,19 +45473,19 @@ l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___c lean_mark_persistent(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___closed__1); l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___closed__2 = _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___closed__2(); lean_mark_persistent(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___closed__2); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__1 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__1(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__1); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__2 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__2(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__2); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__3 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__3(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__3); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__4 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__4(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__4); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__5 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__5(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__5); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__6 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__6(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063____closed__6); -if (builtin) {res = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_7063_(lean_io_mk_world()); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__1 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__1(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__1); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__2 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__2(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__2); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__3 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__3(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__3); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__4 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__4(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__4); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__5 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__5(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__5); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__6 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__6(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753____closed__6); +if (builtin) {res = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Inductive___hyg_8753_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_Elab_Command_bootstrap_inductiveCheckResultingUniverse = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Elab_Command_bootstrap_inductiveCheckResultingUniverse); @@ -37008,6 +45582,10 @@ l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__5 lean_mark_persistent(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__5___closed__2); l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__7___boxed__const__1 = _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__7___boxed__const__1(); lean_mark_persistent(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__7___boxed__const__1); +l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__8___closed__1 = _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__8___closed__1(); +lean_mark_persistent(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__8___closed__1); +l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__8___closed__2 = _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__8___closed__2(); +lean_mark_persistent(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__8___closed__2); l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__1 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__1(); lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__1); l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__2 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__2(); @@ -37050,14 +45628,6 @@ l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__20); l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__21 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__21(); lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__21); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__22 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__22(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__22); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__23 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__23(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__23); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__24 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__24(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__24); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__25 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__25(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__25); l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__1 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__1(); lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__1); l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__2 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__2(); @@ -37100,8 +45670,16 @@ l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambd lean_mark_persistent(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__4); l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__5 = _init_l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__5(); lean_mark_persistent(l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__5); -l_Lean_Elab_Command_elabInductiveViews___lambda__4___boxed__const__1 = _init_l_Lean_Elab_Command_elabInductiveViews___lambda__4___boxed__const__1(); -lean_mark_persistent(l_Lean_Elab_Command_elabInductiveViews___lambda__4___boxed__const__1); +l_Lean_Elab_Command_elabInductiveViewsPostprocessing___lambda__2___boxed__const__1 = _init_l_Lean_Elab_Command_elabInductiveViewsPostprocessing___lambda__2___boxed__const__1(); +lean_mark_persistent(l_Lean_Elab_Command_elabInductiveViewsPostprocessing___lambda__2___boxed__const__1); +l_Lean_Elab_Command_elabClassInductive___closed__1 = _init_l_Lean_Elab_Command_elabClassInductive___closed__1(); +lean_mark_persistent(l_Lean_Elab_Command_elabClassInductive___closed__1); +l_Lean_Elab_Command_elabClassInductive___closed__2 = _init_l_Lean_Elab_Command_elabClassInductive___closed__2(); +lean_mark_persistent(l_Lean_Elab_Command_elabClassInductive___closed__2); +l_Lean_Elab_Command_elabClassInductive___closed__3 = _init_l_Lean_Elab_Command_elabClassInductive___closed__3(); +lean_mark_persistent(l_Lean_Elab_Command_elabClassInductive___closed__3); +l_Array_anyMUnsafe_any___at_Lean_Elab_Command_isMutualInductive___spec__1___closed__1 = _init_l_Array_anyMUnsafe_any___at_Lean_Elab_Command_isMutualInductive___spec__1___closed__1(); +lean_mark_persistent(l_Array_anyMUnsafe_any___at_Lean_Elab_Command_isMutualInductive___spec__1___closed__1); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Lean/Elab/LetRec.c b/stage0/stdlib/Lean/Elab/LetRec.c index 89af18c5d592..06d037f686ca 100644 --- a/stage0/stdlib/Lean/Elab/LetRec.c +++ b/stage0/stdlib/Lean/Elab/LetRec.c @@ -26,6 +26,7 @@ static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_LetRec_0__ lean_object* l_Lean_MapDeclarationExtension_insert___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__18___closed__4; LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_registerLetRecsToLift___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__7___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); lean_object* l_Lean_mkAppN(lean_object*, lean_object*); @@ -70,14 +71,11 @@ lean_object* l_Lean_replaceRef(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_elabLetRec__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__19___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Syntax_getPos_x3f(lean_object*, uint8_t); lean_object* lean_array_fget(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__18___lambda__2___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__23___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Syntax_getTailPos_x3f(lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Elab_elabAttrs___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__17___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_registerLetRecsToLift___spec__2___boxed(lean_object**); lean_object* l_Lean_Expr_fvarId_x21(lean_object*); lean_object* l_Lean_Elab_logException___at_Lean_Elab_Term_exceptionToSorry___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__22___closed__2; @@ -116,6 +114,7 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabLetRec lean_object* l_List_appendTR___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__27(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__22___closed__6; +static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__1; size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__20___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_expandOptDocComment_x3f___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__1___closed__2; @@ -131,6 +130,8 @@ lean_object* l_Lean_ResolveName_resolveNamespace(lean_object*, lean_object*, lea lean_object* l_Array_unzip___rarg(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_registerLetRecsToLift___spec__1___lambda__1___boxed(lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofSyntax(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___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_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__22___closed__3; lean_object* l_Lean_Elab_Term_expandOptType(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -145,14 +146,15 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_ static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__18___lambda__2___closed__4; static lean_object* l_Lean_Elab_expandOptDocComment_x3f___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__1___closed__4; lean_object* l_outOfBounds___rarg(lean_object*); +lean_object* l_Lean_Elab_Term_mkTermInfo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Term_expandDeclId___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_expandOptDocComment_x3f___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__26(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_registerLetRecsToLift___spec__2___boxed(lean_object**); lean_object* l_List_forM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__7___lambda__3___closed__3; lean_object* l_Lean_Syntax_getOptional_x3f(lean_object*); @@ -166,15 +168,18 @@ lean_object* l_Lean_Name_append(lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_getDeclName_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__27___lambda__1___closed__1; static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__7___lambda__4___closed__4; +static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__3; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__27___lambda__4___closed__3; extern lean_object* l_Lean_instInhabitedExpr; LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__7___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__18___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getSepArgs(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_name_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); @@ -183,15 +188,17 @@ static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_Le lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__7___lambda__3___closed__5; uint8_t l_Lean_Syntax_matchesNull(lean_object*, lean_object*); +static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__2; lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_mkFreshExprMVarImpl(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_isIdent(lean_object*); lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_elabLetRec__1___closed__1; static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__18___lambda__2___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Term_elabLetRec_declRange__1___closed__4; static lean_object* l_Lean_Elab_expandOptDocComment_x3f___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Std_Format_defWidth; LEAN_EXPORT lean_object* l___private_Lean_Elab_LetRec_0__Lean_Elab_Term_registerLetRecsToLift(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_LetRec_0__Lean_Elab_Term_withAuxLocalDecls_loop___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -204,7 +211,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_LetRec_0_ uint8_t l_Lean_Environment_contains(lean_object*, lean_object*); static lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__15___rarg___closed__2; LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___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_elabAttr___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__18(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_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__1___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -225,8 +231,8 @@ static lean_object* l___regBuiltin_Lean_Elab_Term_elabLetRec_declRange__1___clos LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__21(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__7___lambda__3___closed__4; lean_object* l_Lean_Elab_Term_addLocalVarInfo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__20(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_registerLetRecsToLift___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__18___lambda__1___boxed(lean_object*); @@ -260,7 +266,9 @@ lean_object* lean_nat_sub(lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__7___lambda__4___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_elabDeclAttrs___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__18___closed__5; +lean_object* l_Lean_Syntax_getRange_x3f(lean_object*, uint8_t); static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__7___lambda__3___closed__2; +lean_object* l_Lean_Elab_Term_withInfoContext_x27(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__27___lambda__5___closed__10; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__21___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_LetRec_0__Lean_Elab_Term_withAuxLocalDecls_loop(lean_object*); @@ -275,7 +283,6 @@ lean_object* lean_array_mk(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_elabAttrs___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__17(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__27___lambda__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_throwErrorAt___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__25___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_addAuxDeclarationRanges___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); static lean_object* l___regBuiltin_Lean_Elab_Term_elabLetRec_declRange__1___closed__6; static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__7___lambda__3___closed__1; @@ -318,7 +325,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_LetRec_ static lean_object* l___regBuiltin_Lean_Elab_Term_elabLetRec__1___closed__6; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); lean_object* l_Lean_MessageData_ofName(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__27___lambda__5___closed__7; static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__18___closed__6; LEAN_EXPORT lean_object* l___private_Lean_Elab_LetRec_0__Lean_Elab_Term_withAuxLocalDecls_loop___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -332,7 +339,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_El LEAN_EXPORT lean_object* l___private_Lean_Elab_LetRec_0__Lean_Elab_Term_registerLetRecsToLift___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_ReaderT_pure___at_Lean_Elab_liftMacroM___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_elabAttr___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__18___lambda__1(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__27___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Binders_0__Lean_Elab_Term_elabBinderViews_loop___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__7___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -681,237 +687,146 @@ return x_56; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_9; uint8_t x_10; lean_object* x_11; lean_object* x_12; -x_9 = lean_ctor_get(x_6, 1); -lean_inc(x_9); -lean_dec(x_6); -x_10 = 0; -x_11 = l_Lean_Syntax_getPos_x3f(x_1, x_10); -x_12 = l_Lean_Syntax_getTailPos_x3f(x_1, x_10); -if (lean_obj_tag(x_11) == 0) +uint8_t x_9; lean_object* x_10; +x_9 = 0; +x_10 = l_Lean_Syntax_getRange_x3f(x_1, x_9); +if (lean_obj_tag(x_10) == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_unsigned_to_nat(0u); -lean_inc(x_9); -x_14 = l_Lean_FileMap_toPosition(x_9, x_13); -lean_inc(x_14); -x_15 = l_Lean_FileMap_leanPosToLspPos(x_9, x_14); -if (lean_obj_tag(x_12) == 0) +lean_object* x_11; lean_object* x_12; +lean_dec(x_6); +x_11 = lean_box(0); +x_12 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_11); +lean_ctor_set(x_12, 1, x_8); +return x_12; +} +else { -uint8_t x_16; -lean_dec(x_9); -x_16 = !lean_is_exclusive(x_15); -if (x_16 == 0) +uint8_t x_13; +x_13 = !lean_is_exclusive(x_10); +if (x_13 == 0) { -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_15, 1); -x_18 = lean_ctor_get(x_15, 0); +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_14 = lean_ctor_get(x_10, 0); +x_15 = lean_ctor_get(x_6, 1); +lean_inc(x_15); +lean_dec(x_6); +x_16 = lean_ctor_get(x_14, 0); +lean_inc(x_16); +lean_inc(x_15); +x_17 = l_Lean_FileMap_toPosition(x_15, x_16); +lean_dec(x_16); +x_18 = lean_ctor_get(x_14, 1); +lean_inc(x_18); +lean_dec(x_14); +lean_inc(x_15); +x_19 = l_Lean_FileMap_toPosition(x_15, x_18); lean_dec(x_18); lean_inc(x_17); -lean_inc(x_14); -x_19 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_19, 0, x_14); -lean_ctor_set(x_19, 1, x_17); -lean_ctor_set(x_19, 2, x_14); -lean_ctor_set(x_19, 3, x_17); -lean_ctor_set(x_15, 1, x_8); -lean_ctor_set(x_15, 0, x_19); -return x_15; -} -else +x_20 = l_Lean_FileMap_leanPosToLspPos(x_15, x_17); +x_21 = !lean_is_exclusive(x_20); +if (x_21 == 0) { -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_15, 1); -lean_inc(x_20); +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_22 = lean_ctor_get(x_20, 1); +x_23 = lean_ctor_get(x_20, 0); +lean_dec(x_23); +lean_inc(x_19); +x_24 = l_Lean_FileMap_leanPosToLspPos(x_15, x_19); lean_dec(x_15); -lean_inc(x_20); -lean_inc(x_14); -x_21 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_21, 0, x_14); -lean_ctor_set(x_21, 1, x_20); -lean_ctor_set(x_21, 2, x_14); -lean_ctor_set(x_21, 3, x_20); -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_21); -lean_ctor_set(x_22, 1, x_8); -return x_22; -} +x_25 = lean_ctor_get(x_24, 1); +lean_inc(x_25); +lean_dec(x_24); +x_26 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_26, 0, x_17); +lean_ctor_set(x_26, 1, x_22); +lean_ctor_set(x_26, 2, x_19); +lean_ctor_set(x_26, 3, x_25); +lean_ctor_set(x_10, 0, x_26); +lean_ctor_set(x_20, 1, x_8); +lean_ctor_set(x_20, 0, x_10); +return x_20; } else { -uint8_t x_23; -x_23 = !lean_is_exclusive(x_15); -if (x_23 == 0) -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_24 = lean_ctor_get(x_15, 1); -x_25 = lean_ctor_get(x_15, 0); -lean_dec(x_25); -x_26 = lean_ctor_get(x_12, 0); -lean_inc(x_26); -lean_dec(x_12); -lean_inc(x_9); -x_27 = l_Lean_FileMap_toPosition(x_9, x_26); -lean_dec(x_26); +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_27 = lean_ctor_get(x_20, 1); lean_inc(x_27); -x_28 = l_Lean_FileMap_leanPosToLspPos(x_9, x_27); -lean_dec(x_9); +lean_dec(x_20); +lean_inc(x_19); +x_28 = l_Lean_FileMap_leanPosToLspPos(x_15, x_19); +lean_dec(x_15); x_29 = lean_ctor_get(x_28, 1); lean_inc(x_29); lean_dec(x_28); x_30 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_30, 0, x_14); -lean_ctor_set(x_30, 1, x_24); -lean_ctor_set(x_30, 2, x_27); +lean_ctor_set(x_30, 0, x_17); +lean_ctor_set(x_30, 1, x_27); +lean_ctor_set(x_30, 2, x_19); lean_ctor_set(x_30, 3, x_29); -lean_ctor_set(x_15, 1, x_8); -lean_ctor_set(x_15, 0, x_30); -return x_15; +lean_ctor_set(x_10, 0, x_30); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_10); +lean_ctor_set(x_31, 1, x_8); +return x_31; +} } else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_31 = lean_ctor_get(x_15, 1); -lean_inc(x_31); -lean_dec(x_15); -x_32 = lean_ctor_get(x_12, 0); +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_32 = lean_ctor_get(x_10, 0); lean_inc(x_32); -lean_dec(x_12); -lean_inc(x_9); -x_33 = l_Lean_FileMap_toPosition(x_9, x_32); +lean_dec(x_10); +x_33 = lean_ctor_get(x_6, 1); +lean_inc(x_33); +lean_dec(x_6); +x_34 = lean_ctor_get(x_32, 0); +lean_inc(x_34); +lean_inc(x_33); +x_35 = l_Lean_FileMap_toPosition(x_33, x_34); +lean_dec(x_34); +x_36 = lean_ctor_get(x_32, 1); +lean_inc(x_36); lean_dec(x_32); lean_inc(x_33); -x_34 = l_Lean_FileMap_leanPosToLspPos(x_9, x_33); -lean_dec(x_9); -x_35 = lean_ctor_get(x_34, 1); +x_37 = l_Lean_FileMap_toPosition(x_33, x_36); +lean_dec(x_36); lean_inc(x_35); -lean_dec(x_34); -x_36 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_36, 0, x_14); -lean_ctor_set(x_36, 1, x_31); -lean_ctor_set(x_36, 2, x_33); -lean_ctor_set(x_36, 3, x_35); -x_37 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_37, 0, x_36); -lean_ctor_set(x_37, 1, x_8); -return x_37; -} -} -} -else -{ -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_11, 0); -lean_inc(x_38); -lean_dec(x_11); -lean_inc(x_9); -x_39 = l_Lean_FileMap_toPosition(x_9, x_38); -lean_dec(x_38); -lean_inc(x_39); -x_40 = l_Lean_FileMap_leanPosToLspPos(x_9, x_39); -if (lean_obj_tag(x_12) == 0) -{ -uint8_t x_41; -lean_dec(x_9); -x_41 = !lean_is_exclusive(x_40); -if (x_41 == 0) -{ -lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_ctor_get(x_40, 1); -x_43 = lean_ctor_get(x_40, 0); -lean_dec(x_43); -lean_inc(x_42); +x_38 = l_Lean_FileMap_leanPosToLspPos(x_33, x_35); +x_39 = lean_ctor_get(x_38, 1); lean_inc(x_39); -x_44 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_44, 0, x_39); -lean_ctor_set(x_44, 1, x_42); -lean_ctor_set(x_44, 2, x_39); -lean_ctor_set(x_44, 3, x_42); -lean_ctor_set(x_40, 1, x_8); -lean_ctor_set(x_40, 0, x_44); -return x_40; -} -else -{ -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_40, 1); -lean_inc(x_45); -lean_dec(x_40); -lean_inc(x_45); -lean_inc(x_39); -x_46 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_46, 0, x_39); -lean_ctor_set(x_46, 1, x_45); -lean_ctor_set(x_46, 2, x_39); -lean_ctor_set(x_46, 3, x_45); -x_47 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_47, 0, x_46); -lean_ctor_set(x_47, 1, x_8); -return x_47; -} -} -else -{ -uint8_t x_48; -x_48 = !lean_is_exclusive(x_40); -if (x_48 == 0) -{ -lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_49 = lean_ctor_get(x_40, 1); -x_50 = lean_ctor_get(x_40, 0); -lean_dec(x_50); -x_51 = lean_ctor_get(x_12, 0); -lean_inc(x_51); -lean_dec(x_12); -lean_inc(x_9); -x_52 = l_Lean_FileMap_toPosition(x_9, x_51); -lean_dec(x_51); -lean_inc(x_52); -x_53 = l_Lean_FileMap_leanPosToLspPos(x_9, x_52); -lean_dec(x_9); -x_54 = lean_ctor_get(x_53, 1); -lean_inc(x_54); -lean_dec(x_53); -x_55 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_55, 0, x_39); -lean_ctor_set(x_55, 1, x_49); -lean_ctor_set(x_55, 2, x_52); -lean_ctor_set(x_55, 3, x_54); -lean_ctor_set(x_40, 1, x_8); -lean_ctor_set(x_40, 0, x_55); -return x_40; +if (lean_is_exclusive(x_38)) { + lean_ctor_release(x_38, 0); + lean_ctor_release(x_38, 1); + x_40 = x_38; +} else { + lean_dec_ref(x_38); + x_40 = lean_box(0); } -else -{ -lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_56 = lean_ctor_get(x_40, 1); -lean_inc(x_56); -lean_dec(x_40); -x_57 = lean_ctor_get(x_12, 0); -lean_inc(x_57); -lean_dec(x_12); -lean_inc(x_9); -x_58 = l_Lean_FileMap_toPosition(x_9, x_57); -lean_dec(x_57); -lean_inc(x_58); -x_59 = l_Lean_FileMap_leanPosToLspPos(x_9, x_58); -lean_dec(x_9); -x_60 = lean_ctor_get(x_59, 1); -lean_inc(x_60); -lean_dec(x_59); -x_61 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_61, 0, x_39); -lean_ctor_set(x_61, 1, x_56); -lean_ctor_set(x_61, 2, x_58); -lean_ctor_set(x_61, 3, x_60); -x_62 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_62, 0, x_61); -lean_ctor_set(x_62, 1, x_8); -return x_62; +lean_inc(x_37); +x_41 = l_Lean_FileMap_leanPosToLspPos(x_33, x_37); +lean_dec(x_33); +x_42 = lean_ctor_get(x_41, 1); +lean_inc(x_42); +lean_dec(x_41); +x_43 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_43, 0, x_35); +lean_ctor_set(x_43, 1, x_39); +lean_ctor_set(x_43, 2, x_37); +lean_ctor_set(x_43, 3, x_42); +x_44 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_44, 0, x_43); +if (lean_is_scalar(x_40)) { + x_45 = lean_alloc_ctor(0, 2, 0); +} else { + x_45 = x_40; } +lean_ctor_set(x_45, 0, x_44); +lean_ctor_set(x_45, 1, x_8); +return x_45; } } } @@ -1355,45 +1270,123 @@ return x_116; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +lean_object* x_11; lean_object* x_12; lean_inc(x_8); -x_11 = l_Lean_Elab_getDeclarationRange___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__5(x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Lean_Elab_getDeclarationRange_x3f___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__5(x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10); x_12 = lean_ctor_get(x_11, 0); lean_inc(x_12); -x_13 = lean_ctor_get(x_11, 1); -lean_inc(x_13); -lean_dec(x_11); -lean_inc(x_8); -x_14 = l_Lean_Elab_getDeclarationRange___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__5(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); -x_15 = !lean_is_exclusive(x_14); -if (x_15 == 0) +if (lean_obj_tag(x_12) == 0) { -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_14, 0); -x_17 = lean_ctor_get(x_14, 1); -lean_ctor_set(x_14, 1, x_16); -lean_ctor_set(x_14, 0, x_12); -x_18 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__6(x_1, x_14, x_4, x_5, x_6, x_7, x_8, x_9, x_17); +uint8_t x_13; lean_dec(x_8); +lean_dec(x_1); +x_13 = !lean_is_exclusive(x_11); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_11, 0); +lean_dec(x_14); +x_15 = lean_box(0); +lean_ctor_set(x_11, 0, x_15); +return x_11; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_11, 1); +lean_inc(x_16); +lean_dec(x_11); +x_17 = lean_box(0); +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set(x_18, 1, x_16); return x_18; } +} else { lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_19 = lean_ctor_get(x_14, 0); -x_20 = lean_ctor_get(x_14, 1); -lean_inc(x_20); +x_19 = lean_ctor_get(x_11, 1); lean_inc(x_19); -lean_dec(x_14); -x_21 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_21, 0, x_12); -lean_ctor_set(x_21, 1, x_19); -x_22 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__6(x_1, x_21, x_4, x_5, x_6, x_7, x_8, x_9, x_20); +lean_dec(x_11); +x_20 = lean_ctor_get(x_12, 0); +lean_inc(x_20); +lean_dec(x_12); +lean_inc(x_8); +x_21 = l_Lean_Elab_getDeclarationRange_x3f___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__5(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_19); +x_22 = lean_ctor_get(x_21, 0); +lean_inc(x_22); +if (lean_obj_tag(x_22) == 0) +{ +uint8_t x_23; +x_23 = !lean_is_exclusive(x_21); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_21, 1); +x_25 = lean_ctor_get(x_21, 0); +lean_dec(x_25); +lean_inc(x_20); +lean_ctor_set(x_21, 1, x_20); +lean_ctor_set(x_21, 0, x_20); +x_26 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__6(x_1, x_21, x_4, x_5, x_6, x_7, x_8, x_9, x_24); lean_dec(x_8); -return x_22; +return x_26; +} +else +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_21, 1); +lean_inc(x_27); +lean_dec(x_21); +lean_inc(x_20); +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_20); +lean_ctor_set(x_28, 1, x_20); +x_29 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__6(x_1, x_28, x_4, x_5, x_6, x_7, x_8, x_9, x_27); +lean_dec(x_8); +return x_29; +} +} +else +{ +uint8_t x_30; +x_30 = !lean_is_exclusive(x_21); +if (x_30 == 0) +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_31 = lean_ctor_get(x_21, 1); +x_32 = lean_ctor_get(x_21, 0); +lean_dec(x_32); +x_33 = lean_ctor_get(x_22, 0); +lean_inc(x_33); +lean_dec(x_22); +lean_ctor_set(x_21, 1, x_33); +lean_ctor_set(x_21, 0, x_20); +x_34 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__6(x_1, x_21, x_4, x_5, x_6, x_7, x_8, x_9, x_31); +lean_dec(x_8); +return x_34; +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_35 = lean_ctor_get(x_21, 1); +lean_inc(x_35); +lean_dec(x_21); +x_36 = lean_ctor_get(x_22, 0); +lean_inc(x_36); +lean_dec(x_22); +x_37 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_37, 0, x_20); +lean_ctor_set(x_37, 1, x_36); +x_38 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__6(x_1, x_37, x_4, x_5, x_6, x_7, x_8, x_9, x_35); +lean_dec(x_8); +return x_38; +} +} } } } @@ -5235,7 +5228,7 @@ lean_inc(x_24); lean_dec(x_23); lean_inc(x_15); lean_inc(x_1); -x_25 = l_Lean_Elab_addAuxDeclarationRanges___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__4(x_1, x_4, x_5, x_11, x_12, x_13, x_14, x_15, x_16, x_24); +x_25 = l_Lean_Elab_addDeclarationRangesFromSyntax___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__4(x_1, x_4, x_5, x_11, x_12, x_13, x_14, x_15, x_16, x_24); x_26 = lean_ctor_get(x_25, 1); lean_inc(x_26); lean_dec(x_25); @@ -6417,11 +6410,11 @@ lean_dec(x_1); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; -x_9 = l_Lean_Elab_getDeclarationRange___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_Elab_getDeclarationRange_x3f___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_7); lean_dec(x_5); lean_dec(x_4); @@ -6445,11 +6438,11 @@ lean_dec(x_3); return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___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_Lean_Elab_addDeclarationRangesFromSyntax___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___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_Elab_addAuxDeclarationRanges___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___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_Elab_addDeclarationRangesFromSyntax___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___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_7); lean_dec(x_6); @@ -7388,7 +7381,44 @@ return x_22; } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("MutualDef", 9, 9); +return x_1; +} +} +static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("body", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__1; +x_2 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__2; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; uint8_t x_12; lean_object* x_13; +x_11 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__3; +x_12 = 0; +lean_inc(x_2); +x_13 = l_Lean_Elab_Term_mkTermInfo(x_11, x_1, x_3, x_2, x_2, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; @@ -7406,7 +7436,7 @@ x_16 = l_Std_Range_forIn_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_ lean_dec(x_2); if (lean_obj_tag(x_16) == 0) { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; x_17 = lean_ctor_get(x_16, 1); lean_inc(x_17); lean_dec(x_16); @@ -7418,17 +7448,26 @@ lean_dec(x_3); x_20 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_20, 0, x_5); x_21 = lean_box(0); +lean_inc(x_19); x_22 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__1), 11, 4); lean_closure_set(x_22, 0, x_19); lean_closure_set(x_22, 1, x_20); lean_closure_set(x_22, 2, x_21); lean_closure_set(x_22, 3, x_4); -x_23 = l_Lean_Elab_Term_withDeclName___rarg(x_18, x_22, x_6, x_7, x_8, x_9, x_10, x_11, x_17); -return x_23; +lean_inc(x_19); +x_23 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___boxed), 10, 2); +lean_closure_set(x_23, 0, x_19); +lean_closure_set(x_23, 1, x_21); +x_24 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withInfoContext_x27), 10, 3); +lean_closure_set(x_24, 0, x_19); +lean_closure_set(x_24, 1, x_22); +lean_closure_set(x_24, 2, x_23); +x_25 = l_Lean_Elab_Term_withDeclName___rarg(x_18, x_24, x_6, x_7, x_8, x_9, x_10, x_11, x_17); +return x_25; } else { -uint8_t x_24; +uint8_t x_26; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -7438,23 +7477,23 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_24 = !lean_is_exclusive(x_16); -if (x_24 == 0) +x_26 = !lean_is_exclusive(x_16); +if (x_26 == 0) { return x_16; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_16, 0); -x_26 = lean_ctor_get(x_16, 1); -lean_inc(x_26); -lean_inc(x_25); +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_16, 0); +x_28 = lean_ctor_get(x_16, 1); +lean_inc(x_28); +lean_inc(x_27); lean_dec(x_16); -x_27 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_26); -return x_27; +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_27); +lean_ctor_set(x_29, 1, x_28); +return x_29; } } } @@ -7492,7 +7531,7 @@ x_18 = lean_array_get_size(x_17); lean_inc(x_18); x_19 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_19, 0, x_18); -x_20 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___boxed), 12, 3); +x_20 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__3___boxed), 12, 3); lean_closure_set(x_20, 0, x_17); lean_closure_set(x_20, 1, x_18); lean_closure_set(x_20, 2, x_13); @@ -7578,11 +7617,25 @@ lean_dec(x_1); return x_16; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; -x_13 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_13 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_1); return x_13; } @@ -7769,7 +7822,7 @@ return x_57; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_registerLetRecsToLift___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_registerLetRecsToLift___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { _start: { lean_object* x_18; uint8_t x_19; @@ -7992,7 +8045,7 @@ lean_dec(x_21); x_24 = lean_array_get_size(x_1); x_25 = lean_mk_empty_array_with_capacity(x_24); x_26 = lean_unsigned_to_nat(0u); -x_27 = l_Array_mapIdxM_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_registerLetRecsToLift___spec__2(x_1, x_2, x_3, x_20, x_22, x_1, x_24, x_26, lean_box(0), x_25, x_4, x_5, x_6, x_7, x_8, x_9, x_23); +x_27 = l_Array_mapFinIdxM_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_registerLetRecsToLift___spec__2(x_1, x_2, x_3, x_20, x_22, x_1, x_24, x_26, lean_box(0), x_25, x_4, x_5, x_6, x_7, x_8, x_9, x_23); lean_dec(x_8); lean_dec(x_6); lean_dec(x_4); @@ -8141,7 +8194,7 @@ lean_dec(x_2); return x_15; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_registerLetRecsToLift___spec__2___boxed(lean_object** _args) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_registerLetRecsToLift___spec__2___boxed(lean_object** _args) { lean_object* x_1 = _args[0]; lean_object* x_2 = _args[1]; lean_object* x_3 = _args[2]; @@ -8162,7 +8215,7 @@ lean_object* x_17 = _args[16]; _start: { lean_object* x_18; -x_18 = l_Array_mapIdxM_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_registerLetRecsToLift___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +x_18 = l_Array_mapFinIdxM_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_registerLetRecsToLift___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); @@ -9106,6 +9159,12 @@ l_Array_forInUnsafe_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLet lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__27___lambda__5___closed__10); l_Std_Range_forIn_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__1___closed__1 = _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__1___closed__1(); lean_mark_persistent(l_Std_Range_forIn_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__1___closed__1); +l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__1 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__1(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__1); +l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__2 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__2(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__2); +l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__3 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__3(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__3); l___regBuiltin_Lean_Elab_Term_elabLetRec__1___closed__1 = _init_l___regBuiltin_Lean_Elab_Term_elabLetRec__1___closed__1(); lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_elabLetRec__1___closed__1); l___regBuiltin_Lean_Elab_Term_elabLetRec__1___closed__2 = _init_l___regBuiltin_Lean_Elab_Term_elabLetRec__1___closed__2(); diff --git a/stage0/stdlib/Lean/Elab/Match.c b/stage0/stdlib/Lean/Elab/Match.c index f14a659ed659..23d781e79d36 100644 --- a/stage0/stdlib/Lean/Elab/Match.c +++ b/stage0/stdlib/Lean/Elab/Match.c @@ -173,7 +173,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_withPatte LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_getMatchGeneralizing_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitLet___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__6(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); 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*); -uint8_t l_Array_contains___at_Lean_findField_x3f___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrsWitMatchType___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitLet___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__6___lambda__1(lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_ToDepElimPattern_main___rarg___lambda__2___closed__3; @@ -951,6 +950,7 @@ static lean_object* l___regBuiltin_Lean_Elab_Term_elabNoMatch_declRange__1___clo 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_Meta_transform_visit_visitLet___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(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__4___boxed(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_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*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_precheckMatch___spec__4(size_t, size_t, lean_object*); @@ -38340,7 +38340,7 @@ lean_inc(x_21); lean_dec(x_19); x_22 = l_Lean_LocalDecl_userName(x_20); lean_dec(x_20); -x_23 = l_Array_contains___at_Lean_findField_x3f___spec__1(x_6, x_22); +x_23 = l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(x_6, x_22); if (x_23 == 0) { lean_object* x_24; lean_object* x_25; uint8_t x_26; @@ -38490,7 +38490,7 @@ lean_inc(x_21); lean_dec(x_19); x_22 = l_Lean_LocalDecl_userName(x_20); lean_dec(x_20); -x_23 = l_Array_contains___at_Lean_findField_x3f___spec__1(x_6, x_22); +x_23 = l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(x_6, x_22); if (x_23 == 0) { lean_object* x_24; lean_object* x_25; uint8_t x_26; diff --git a/stage0/stdlib/Lean/Elab/MutualDef.c b/stage0/stdlib/Lean/Elab/MutualDef.c index c30e4edeaa12..e52ee75d4a85 100644 --- a/stage0/stdlib/Lean/Elab/MutualDef.c +++ b/stage0/stdlib/Lean/Elab/MutualDef.c @@ -44,13 +44,11 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_getAl LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapMAux___at_Lean_Elab_Term_elabMutualDef___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_mapMUnsafe_map___at_Lean_LocalContext_getFVars___spec__1(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_checkKinds(uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__13; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkFreeVarMap___spec__5___rarg___closed__3; static lean_object* l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualDef___spec__4___closed__3; lean_object* l_Lean_MapDeclarationExtension_insert___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___lambda__2___closed__11; LEAN_EXPORT lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_declValToTerminationHint___spec__1___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef_go___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_Meta_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___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_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosureFor___spec__5(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosures___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -69,17 +67,17 @@ lean_object* l_Lean_mkAppN(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__5___boxed(lean_object**); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_registerFailedToInferDefTypeInfo___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_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__5___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___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* l_Lean_Elab_CommandContextInfo_save___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_cleanupOfNat___lambda__2___closed__3; static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__4___closed__3; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__4; static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__5___lambda__2___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_checkKinds___lambda__1(uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_checkKinds___lambda__1___closed__2; static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__3___closed__8; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__5___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__6___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__9; static lean_object* l_Lean_Elab_instInhabitedDefViewElabHeader___closed__3; -static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__10; static lean_object* l_Lean_Elab_instInhabitedDefViewElabHeader___closed__6; LEAN_EXPORT lean_object* l_Array_erase___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkClosureForAux___spec__2___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_processDeriving___spec__1(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -96,25 +94,23 @@ static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeader LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_FixPoint_merge(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders_mkBodyTask(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_MutualDef___hyg_6346____closed__3; -static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__7; lean_object* l_Lean_Elab_Command_runTermElabM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef_go___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkClosureForAux___closed__2; LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__6; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders_mkTacTask___closed__5; extern lean_object* l_Lean_declRangeExt; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check___lambda__2___closed__5; static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_declValToTerminationHint___spec__1___lambda__3___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__5___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosureFor___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__4___closed__2; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_cleanupOfNat___lambda__2___closed__1; static lean_object* l_Nat_foldM_loop___at_Lean_Elab_Term_MutualClosure_pushMain___spec__1___closed__1; lean_object* l_Lean_throwError___at_Lean_Elab_Term_mkAuxName___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_linter_unusedSectionVars; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__1(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__4; extern lean_object* l_Lean_Elab_Tactic_instInhabitedTacticParsedSnapshot; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__8___boxed(lean_object**); @@ -122,7 +118,6 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Mutua lean_object* l_Lean_Language_Snapshot_Diagnostics_ofMessageLog(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_cleanupOfNat___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_getMax_x3f___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_pickMaxFVar_x3f___spec__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Language_withAlwaysResolvedPromises___at_Lean_Elab_Term_elabMutualDef_go___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__5___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Language_DynamicSnapshot_toTyped_x3f___rarg(lean_object*, lean_object*); lean_object* l_Lean_Meta_isProp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -152,9 +147,8 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_Mutua LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabMutualDef_processDeriving(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__12___lambda__2___closed__11; lean_object* l_Lean_MessageData_joinSep(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__3___boxed(lean_object**); +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_uint64_to_usize(uint64_t); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__11; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__5___rarg___lambda__2(lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosures___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isAppOfArity(lean_object*, lean_object*, lean_object*); @@ -167,7 +161,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_clean static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__4___rarg___closed__1; lean_object* l_Lean_Elab_logException___at_Lean_Elab_Command_elabCommand___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_toString(lean_object*, uint8_t, lean_object*); -static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__9; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosures(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getId(lean_object*); @@ -175,7 +168,7 @@ static lean_object* l_Nat_foldM_loop___at_Lean_Elab_Term_MutualClosure_pushMain_ lean_object* l_Lean_Elab_Term_elabTermEnsuringType(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__6___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_sort___override(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofList(lean_object*); lean_object* l_Lean_PersistentArray_push___rarg(lean_object*, lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); @@ -194,20 +187,21 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Mutua LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_checkLetRecsToLiftTypes___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_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkClosureForAux___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__7___boxed(lean_object**); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__15(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_MutualDef_0__Lean_Elab_Term_check___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_mk_array(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__6___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___closed__4; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__5(lean_object*); -static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__3; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check___lambda__4___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__2(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); +static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__7___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_deprecated_oldSectionVars; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_checkModifiers___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosureFor___spec__3(lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__3___closed__1; uint8_t l_Array_contains___at___private_Lean_Class_0__Lean_checkOutParam___spec__1(lean_object*, lean_object*); lean_object* l_Lean_Syntax_getArgs(lean_object*); @@ -228,7 +222,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_MutualClosure_Replacement_apply___lamb static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkClosureForAux___closed__5; lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_shareCommonPreDefs(lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Syntax_getPos_x3f(lean_object*, uint8_t); lean_object* l_Lean_Expr_bvar___override(lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__18(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -238,12 +231,12 @@ static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0_ lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_levelMVarToParamTypesPreDecls___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__12___boxed(lean_object**); -lean_object* l_Lean_Syntax_getTailPos_x3f(lean_object*, uint8_t); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_cleanupOfNat___lambda__3___closed__2; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_getPendingMVarErrorMessage___closed__1; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosures___spec__11___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosures___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_TSepArray_getElems___rarg(lean_object*); +static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__14; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabMutualDef___spec__12(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_fvarId_x21(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__12___lambda__2___closed__9; @@ -261,6 +254,7 @@ static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeader LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef___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*); static lean_object* l_Lean_Elab_Command_elabMutualDef___lambda__3___closed__5; LEAN_EXPORT lean_object* l_Lean_RBNode_fold___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkFreeVarMap___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef_go___spec__17(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_getPendingMVarErrorMessage___closed__2; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabMutualDef___spec__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__5___lambda__3___closed__4; @@ -271,18 +265,20 @@ LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Elab_Command_elabM LEAN_EXPORT lean_object* l_Lean_Meta_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__12___lambda__1___boxed(lean_object**); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosures___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__4(lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___at_Lean_Elab_Term_elabMutualDef_go___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_MutualClosure_main___spec__3(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__5___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__5___lambda__2___closed__1; +static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__3; static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__18___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef___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___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_checkModifiers___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_Term_initFn____x40_Lean_Elab_MutualDef___hyg_6307____closed__6; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__3; LEAN_EXPORT uint8_t l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_isExample(lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars_collectUsed___spec__5___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars_collectUsed___spec__6(lean_object*, lean_object*, size_t, size_t); -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_node5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars_collectUsed___spec__4(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_MutualDef___hyg_6346____closed__2; @@ -311,20 +307,23 @@ static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_cleanupOfN static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___lambda__2___closed__5; static lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3___closed__5; uint8_t l_Lean_MapDeclarationExtension_contains___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__5; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars___spec__1___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_declValToTerminationHint___spec__1___lambda__1___closed__3; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__5; lean_object* l_Lean_RBNode_findCore___at_Lean_Meta_mkGeneralizationForbiddenSet_visit___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosures___spec__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_List_any___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___lambda__2(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__4(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_MutualClosure_main___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_head_x21___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_cleanupOfNat___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__12___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Term_elabMutualDef_go___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_MutualClosure_Replacement_apply(lean_object*, lean_object*); static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__6___lambda__5___closed__7; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__13; LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_isMultiConstant_x3f___spec__2(lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___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___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -347,23 +346,25 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_level lean_object* l_Lean_Core_getAndEmptyMessageLog___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualDef___spec__4___closed__5; LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__6___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_levelMVarToParamHeaders_process(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_declValToTerm(lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Elab_DefKind_isExample(uint8_t); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_levelMVarToParamHeaders___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__1; lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Intro_0__Lean_Meta_introNImp___spec__1(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_instantiateMVarsAtLetRecToLift___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_appArg_x21(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_FVarId_findDecl_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Elab_Command_elabMutualDef___spec__10___lambda__1___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_MutualDef___hyg_6307____closed__4; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476_(lean_object*); lean_object* l_Lean_Elab_Term_elabBindersEx___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__1; +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkClosureForAux___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_checkLetRecsToLiftTypes(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_index(lean_object*); @@ -379,8 +380,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_MutualClosure_FixPoint_run___boxed(lea static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_processDeriving___spec__1___closed__1; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars_collectUsed___spec__4___closed__3; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_cleanupOfNat___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Term_elabMutualDef_go___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__3; static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__5___lambda__3___closed__5; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders_mkTacTask___closed__6; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_checkModifiers___closed__2; @@ -394,11 +393,11 @@ LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_MutualDef_0_ static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_declValToTerminationHint___spec__1___lambda__3___closed__2; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders_getBodyTerm_x3f___closed__2; lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___boxed(lean_object**); LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__5___lambda__3___closed__3; LEAN_EXPORT lean_object* l_Lean_RBNode_fold___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_pushNewVars___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_filterMapM___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__7; lean_object* lean_io_promise_resolve(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_collectUsed___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -412,7 +411,6 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Mutua LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_FixPoint_fixpoint(lean_object*); lean_object* l_Lean_Elab_Term_expandWhereDeclsOpt(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_getPendingMVarErrorMessage___closed__4; -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_withLCtx___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -429,6 +427,7 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDe LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__5___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_reverse___rarg(lean_object*); +static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__12; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_levelMVarToParamHeaders_process___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_List_elem___at_Lean_addAliasEntry___spec__16(lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___lambda__1(lean_object*, size_t, lean_object*); @@ -444,7 +443,6 @@ lean_object* l_Lean_LocalDecl_setUserName(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef___spec__10(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Array_contains___at_Lean_Meta_setMVarUserNamesAt___spec__1(lean_object*, lean_object*); lean_object* lean_st_ref_take(lean_object*, lean_object*); -static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__1; static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_declValToTerminationHint___spec__1___lambda__1___closed__4; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__3___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars_getFVars___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -453,6 +451,7 @@ static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_Mu LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosureFor___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_getDeclarationSelectionRef(lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_find___at_Lean_Elab_Term_MutualClosure_isApplicable___spec__1(lean_object*, lean_object*); +static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__7; LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__6___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_checkModifiers___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_realizeGlobalConstNoOverload(lean_object*, lean_object*, lean_object*, lean_object*); @@ -469,6 +468,7 @@ lean_object* l_Array_unzip___rarg(lean_object*); lean_object* l_Array_feraseIdx___rarg(lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__12___lambda__2___closed__12; lean_object* l_Lean_SourceInfo_fromRef(lean_object*, uint8_t); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__6; LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars___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_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__18___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_checkModifiers(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -477,6 +477,7 @@ lean_object* l_List_findSome_x3f___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__2___rarg___lambda__1(lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__3___closed__5; LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__14___boxed(lean_object**); +static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__5; lean_object* l_Lean_Syntax_node6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_FixPoint_isModified___boxed(lean_object*); uint8_t l_Lean_RBNode_isSingleton___rarg(lean_object*); @@ -486,6 +487,7 @@ lean_object* lean_nat_div(lean_object*, lean_object*); lean_object* lean_io_add_heartbeats(uint64_t, lean_object*); lean_object* l_Lean_mkHole(lean_object*, uint8_t); LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_collectUsed___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Elab_Command_elabMutualDef___spec__10___lambda__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___lambda__2___closed__4; LEAN_EXPORT uint8_t l_List_mapTR_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_getPendingMVarErrorMessage___spec__1___lambda__1(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -500,6 +502,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_Mutua LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_checkKinds___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_registerTraceClass(lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosureFor___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__7; LEAN_EXPORT lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_declValToTerminationHint___spec__1___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__13(lean_object*, lean_object*, lean_object*, lean_object*); @@ -516,14 +519,15 @@ static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check___la LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_processDeriving___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_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars_collectUsed___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*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars_collectUsed___spec__4___closed__4; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef_go___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__12___lambda__2___closed__5; lean_object* l_Lean_CollectFVars_State_addDependencies(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__15; LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_Term_MutualClosure_insertReplacementForLetRecs___spec__1(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_Term_MutualClosure_isApplicable___lambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabMutualDef___spec__13(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_toAttributeKind___boxed(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(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef_go___spec__13(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(lean_object*, lean_object*); lean_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_RBNode_find___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosures___spec__13___boxed(lean_object*, lean_object*); @@ -531,7 +535,6 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualD LEAN_EXPORT lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_declValToTerminationHint___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_List_foldlM___at_Lean_Elab_Term_MutualClosure_pushLetRecs___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* l_Lean_Syntax_getKind(lean_object*); -static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__5; static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_declValToTerminationHint___spec__1___lambda__6___closed__2; lean_object* l_Lean_MessageData_ofFormat(lean_object*); lean_object* l_Lean_PersistentArray_append___rarg(lean_object*, lean_object*); @@ -541,25 +544,26 @@ lean_object* l_Lean_Meta_check(lean_object*, lean_object*, lean_object*, lean_ob static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___closed__1; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef___spec__11(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__12___lambda__2___closed__4; -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__7(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_transform___at_Lean_Meta_zetaReduce___spec__1(lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_FVarId_getDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_outOfBounds___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__15___boxed(lean_object**); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__10; +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Term_elabMutualDef_go___spec__7___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_elabAttrs___at_Lean_Elab_Command_elabMutualDef___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__5___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_MutualDef___hyg_6346_(lean_object*); +lean_object* l_Lean_Elab_Term_mkTermInfo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_indexOfAux___at_Lean_LocalContext_erase___spec__3(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3___closed__4; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosures___spec__7(lean_object*, lean_object*, lean_object*, size_t, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withFunLocalDecls(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_declValToTerminationHint___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosures___spec__4(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__8; lean_object* lean_st_ref_get(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_filterMapM___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualDef___spec__4___closed__1; @@ -572,16 +576,15 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabH LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_MutualClosure_Replacement_apply___lambda__1___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__11; static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__6___lambda__5___closed__3; LEAN_EXPORT lean_object* l_Lean_addTrace___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkClosureForAux___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__18___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withReuseContext___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__13(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getOptional_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabMutualDef_go___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_mk_ref(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_FixPoint_updateUsedVarsOf___lambda__1(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Term_elabMutualDef_go___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_isExample___spec__1(lean_object*, size_t, size_t); LEAN_EXPORT uint8_t l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualDef___spec__4___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__4___rarg___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -593,7 +596,6 @@ LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_Term_MutualClosure_mai static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_cleanupOfNat___lambda__2___closed__4; LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_Term_MutualClosure_main___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___closed__2; -static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualDef___spec__4___lambda__2(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars_collectUsed___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_withSaveInfoContext___at_Lean_Elab_Term_elabMutualDef___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -607,7 +609,6 @@ lean_object* l_Lean_Elab_instantiateMVarsAtPreDecls(lean_object*, lean_object*, lean_object* l_Lean_throwError___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_declValToTerminationHint___spec__1___lambda__1___closed__1; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___lambda__2___closed__6; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_levelMVarToParamHeaders_process___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_pushLocalDecl(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__4___closed__4; @@ -615,17 +616,18 @@ LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_E LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabMutualDef___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabMutualDef_go___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues(lean_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_elabMutualDef_go___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*); uint8_t l_Lean_Syntax_isMissing(lean_object*); LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__6___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders_mkTacTask___closed__2; -static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5___closed__1; static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__6___lambda__5___closed__4; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__2; extern lean_object* l_Lean_levelZero; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__5___closed__4; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__1___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars_collectUsed___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__2(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___lambda__2___closed__2; LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__6___lambda__1___boxed(lean_object**); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__12___lambda__2___closed__13; @@ -637,7 +639,8 @@ LEAN_EXPORT lean_object* l_Lean_RBNode_fold___at___private_Lean_Elab_MutualDef_0 lean_object* l_Lean_Elab_InfoTree_substitute(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_checkModifiers___lambda__2___closed__2; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders_mkTacTask___lambda__1___closed__4; -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__11; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders_getBodyTerm_x3f___closed__5; LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_cleanupOfNat___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkFreeVarMap___spec__5(lean_object*); @@ -690,7 +693,6 @@ static lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_MutualDef_0__ static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__3___closed__3; static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_MutualDef___hyg_6307____closed__5; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_MutualClosure_main___spec__2(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__2; lean_object* l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_erase___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkClosureForAux___spec__2(lean_object*, lean_object*); lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); @@ -705,10 +707,10 @@ uint8_t l_Lean_Syntax_matchesNull(lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__12___lambda__2___closed__6; lean_object* l_Lean_Meta_Closure_mkForall(lean_object*, lean_object*); lean_object* l_Lean_Meta_lambdaTelescope___at___private_Lean_Elab_PreDefinition_WF_Fix_0__Lean_Elab_WF_processSumCasesOn___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_Elab_Term_elabMutualDef_go___spec__17(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders_mkTacTask___lambda__1___closed__3; extern lean_object* l_Lean_Elab_instInhabitedDefView; static lean_object* l_Lean_Elab_Command_elabMutualDef___lambda__3___closed__2; +LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars_collectUsed___spec__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabMutualDef___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_isIdent(lean_object*); @@ -746,11 +748,15 @@ lean_object* l_Lean_Elab_Term_withAutoBoundImplicitForbiddenPred___rarg(lean_obj extern lean_object* l_Std_Format_defWidth; LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_declValToTerminationHint___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_instInhabitedDefViewElabHeader___closed__2; +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Term_elabMutualDef_go___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_getZetaDeltaFVarIds___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_MutualClosure_getModifiersForLetRecs___spec__2___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabMutualDef_go___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_FixPoint_getUsedFVarsMap___boxed(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosures___spec__7___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosures___spec__8(lean_object*, lean_object*, size_t, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___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* l_Lean_Meta_Closure_mkLambda(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_MutualClosure_pushLetRecs___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___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*); @@ -760,6 +766,8 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualD lean_object* l_Lean_MVarId_assign___at_Lean_Elab_Term_exprToSyntax___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_pickMaxFVar_x3f___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualDef___spec__4___closed__6; +lean_object* lean_mk_thunk(lean_object*); +LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders_getBodyTerm_x3f___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_MutualClosure_isApplicable___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_MutualClosure_getKindForLetRecs___boxed(lean_object*); @@ -786,8 +794,8 @@ lean_object* l_Lean_instantiateMVars___at___private_Lean_Meta_Basic_0__Lean_Meta static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__12___lambda__2___closed__8; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__4___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__5___lambda__4___closed__1; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__12; extern lean_object* l_Lean_Elab_TerminationHints_none; +static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__6; LEAN_EXPORT lean_object* l_Array_filterMapM___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__6(lean_object*, size_t, size_t, lean_object*); @@ -805,6 +813,7 @@ lean_object* l_Lean_LocalDecl_userName(lean_object*); lean_object* l_Lean_Syntax_node4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__5___closed__1; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_registerFailedToInferDefTypeInfo___closed__2; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___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_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders_mkTacTask___closed__4; extern lean_object* l_Lean_Elab_instTypeNameDefsParsedSnapshot; @@ -814,20 +823,19 @@ LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_E static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_MutualDef___hyg_6307____closed__1; LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__17(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_MutualClosure_main___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__8; +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Term_elabMutualDef_go___spec__7___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_declValToTerminationHint___spec__1___lambda__3___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_cleanupOfNat(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__3___closed__4; +static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__13; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkFreeVarMap___spec__5___rarg___closed__1; static lean_object* l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualDef___spec__4___lambda__2___closed__2; lean_object* l_Lean_FileMap_leanPosToLspPos(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__2(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_TerminationHints_rememberExtraParams(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__5___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__6; -LEAN_EXPORT lean_object* l_Lean_Language_withAlwaysResolvedPromises___at_Lean_Elab_Term_elabMutualDef_go___spec__15(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__12___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Nat_foldM_loop___at_Lean_Elab_Term_MutualClosure_pushMain___spec__1___lambda__1(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Parser_Term_type; @@ -862,11 +870,11 @@ static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check___la LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___boxed__const__1; LEAN_EXPORT lean_object* l_List_foldlM___at_Lean_Elab_Term_MutualClosure_pushLetRecs___spec__1___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_object*); lean_object* l_Lean_Elab_addPreDefinitions(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Language_withAlwaysResolvedPromises___at_Lean_Elab_Term_elabMutualDef_go___spec__16(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_app___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__6___boxed(lean_object**); LEAN_EXPORT lean_object* l_Lean_Elab_withSaveInfoContext___at_Lean_Elab_Term_elabMutualDef___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_CollectMVars_visit(lean_object*, lean_object*); -static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__3; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_declValToTerminationHint___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__5___closed__1; LEAN_EXPORT lean_object* l_Lean_RBNode_fold___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkFreeVarMap___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); @@ -876,7 +884,9 @@ uint8_t l_List_beq___at___private_Lean_Declaration_0__Lean_beqConstantVal____x40 LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__14(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_typeHasRecFun___lambda__2___boxed(lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___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_Elab_Command_elabMutualDef___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Term_elabMutualDef_go___spec__7___closed__2; lean_object* l_Lean_Elab_getResetInfoTrees___at_Lean_Elab_Term_withDeclName___spec__3___rarg(lean_object*, lean_object*); lean_object* l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_getFVarLocalDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -892,7 +902,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_getPe uint8_t lean_nat_dec_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__12___lambda__2___boxed(lean_object**); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef___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_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__10(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabMutualDef_go___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_isTracingEnabledFor___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkClosureForAux___spec__1___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -900,17 +909,13 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabMutualDef(lean_object*, lean_ob LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkClosureFor___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_instantiateMVars___at___private_Lean_Meta_Basic_0__Lean_Meta_isClassApp_x3f___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withFunLocalDecls_loop___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__13; LEAN_EXPORT lean_object* l_Lean_Elab_Term_MutualClosure_pushLetRecs(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___lambda__1___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__7___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabMutualDef___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_cleanupOfNat___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__7; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef_go___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___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___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkClosureForAux___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__2; LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_MutualClosure_getModifiersForLetRecs___spec__3(lean_object*, size_t, size_t); lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_registerFailedToInferDefTypeInfo___closed__1; @@ -928,8 +933,10 @@ LEAN_EXPORT lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_El static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__5___lambda__1___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_getFunName___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__5___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__3; LEAN_EXPORT lean_object* l_Nat_foldM_loop___at_Lean_Elab_Term_MutualClosure_pushMain___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Nat_foldM_loop___at_Lean_Elab_Term_MutualClosure_pushMain___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef_go___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* l_Lean_Syntax_node1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___closed__5; @@ -981,8 +988,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_remov static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_cleanupOfNat___lambda__4___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); -static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__6; -static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__12; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef___spec__7(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalContext_get_x21(lean_object*, lean_object*); @@ -999,18 +1004,16 @@ static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0_ static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_MutualDef___hyg_6307____closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkFreeVarMap___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosures___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_RBNode_find___at_Lean_Elab_Term_MutualClosure_isApplicable___spec__1___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef_go___spec__12(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__3(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__18___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__3___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Elab_Term_withInfoContext_x27(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___lambda__2___closed__3; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__9; lean_object* l_List_iotaTR(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__11___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_declValToTerminationHint___spec__1___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabMutualDef___spec__6(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_getPendingMVarErrorMessage(lean_object*); -static lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__7___closed__1; lean_object* l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders_mkTacTask___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_LocalDecl_binderInfo(lean_object*); @@ -1026,7 +1029,6 @@ extern lean_object* l_Lean_instInhabitedDeclarationRanges; lean_object* lean_erase_macro_scopes(lean_object*); lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabSyntax___spec__14(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Term_elabMatch_elabMatchDefault___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_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef_go___spec__16(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_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosures___spec__15___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 uint8_t l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_isTheorem(lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Elab_Command_elabMutualDef___spec__9___lambda__1(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1039,11 +1041,11 @@ LEAN_EXPORT lean_object* l_Lean_RBNode_fold___at___private_Lean_Elab_MutualDef_0 LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef_go___spec__6(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_reverse___rarg(lean_object*); lean_object* l_Lean_Elab_Term_withAuxDecl___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_MutualDef___hyg_6346____closed__5; LEAN_EXPORT lean_object* l_Lean_Meta_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__15___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withFunLocalDecls_loop___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_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__8; uint8_t l_Lean_Expr_hasSorry(lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars_getFVars___closed__1; lean_object* l_String_intercalate(lean_object*, lean_object*); @@ -1058,7 +1060,6 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualD static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkFreeVarMap___spec__5___rarg___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_FixPoint_fixpoint___boxed(lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check___lambda__6___closed__1; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__1; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_isMultiConstant_x3f___spec__2___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_declValToTerminationHint___spec__1___lambda__1___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_FixPoint_modifyUsedFVars___boxed(lean_object*, lean_object*, lean_object*); @@ -1069,7 +1070,9 @@ uint8_t l_Lean_Syntax_hasMissing(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__5___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__6___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosureFor___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabMutualDef_go(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___boxed(lean_object**); +static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__8; +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__10; lean_object* l_Lean_getDelayedMVarRoot___rarg(lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Elab_Term_instInhabitedLetRecToLift; size_t lean_usize_add(size_t, size_t); @@ -1088,23 +1091,25 @@ static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_MutualDef LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars___spec__2(lean_object*); static lean_object* l_List_mapTR_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_getPendingMVarErrorMessage___spec__2___closed__2; LEAN_EXPORT lean_object* l_List_foldlM___at_Lean_Elab_Term_MutualClosure_pushLetRecs___spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___at_Lean_Elab_Term_elabMutualDef_go___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_withLevelNames___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_mapTR_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_getPendingMVarErrorMessage___spec__1___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___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_array_uget(lean_object*, size_t); LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualDef___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__4; lean_object* l_Lean_Expr_fvar___override(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_array_size(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef___spec__6(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_getPendingMVarErrorMessage___closed__3; -static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__14; LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__6___boxed(lean_object**); static lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_MutualClosure_FixPoint_run(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars_collectUsed___spec__5(lean_object*, lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__5(lean_object*, lean_object*, size_t, size_t, size_t, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_FixPoint_getUsedFVarsMap(lean_object*); lean_object* l_Lean_Language_SnapshotTask_get___rarg(lean_object*); uint8_t l_Lean_Elab_Modifiers_isNonrec(lean_object*); @@ -1113,10 +1118,12 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Mutua static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkClosureForAux___closed__6; lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withUsed___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__15; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__1___rarg___lambda__2(lean_object*, size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_declValToTerminationHint___spec__1___lambda__2___closed__4; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_isExample___spec__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_getFunName___closed__1; +static lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Term_elabMutualDef_go___spec__7___closed__1; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__12___lambda__2___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_MutualClosure_pushMain(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_FixPoint_fixpoint___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); @@ -1138,10 +1145,10 @@ static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_Mu LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_MutualClosure_getModifiersForLetRecs___spec__2(lean_object*, size_t, size_t); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_processDeriving___spec__1___closed__3; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkFreeVarMap___spec__5___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkFreeVarMap___spec__6___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__6; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders_mkTacTask___lambda__1___closed__9; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders_mkTacTask___lambda__1___closed__7; lean_object* lean_string_append(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__6___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_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_object* l_Lean_getAttributeImpl(lean_object*, lean_object*); @@ -1154,11 +1161,11 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualD LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__11___lambda__1___boxed(lean_object**); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_cleanupOfNat___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5___boxed(lean_object**); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__3___rarg___lambda__3(lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__3(size_t, size_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Term_elabMutualDef_go___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__13(lean_object*, size_t, size_t); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars_collectUsed___spec__4___closed__2; 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(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, size_t, size_t, lean_object*); @@ -1184,15 +1191,19 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Mutua LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_isMultiConstant_x3f___boxed(lean_object*); static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__3___closed__9; lean_object* lean_nat_add(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Language_withAlwaysResolvedPromises___at_Lean_Elab_Term_elabMutualDef_go___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_elabTerminationHints___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_declValToTerminationHint___spec__1___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_processDeriving___spec__1___closed__4; +static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__4___boxed(lean_object**); static lean_object* l_Nat_foldM_loop___at_Lean_Elab_Term_MutualClosure_pushMain___spec__1___closed__3; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__12; uint8_t l_Lean_Exception_isRuntime(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___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_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__10; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___lambda__2___closed__9; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___rarg___boxed__const__1; +static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__5; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosures___spec__3(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__4___rarg___lambda__4(lean_object*, size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); @@ -1212,18 +1223,18 @@ LEAN_EXPORT lean_object* l_Array_sequenceMap_loop___at___private_Lean_Elab_Mutua LEAN_EXPORT lean_object* l_Lean_Elab_Term_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___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_object*, lean_object*, lean_object*); lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabSyntax___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__7; lean_object* l_Lean_Elab_fixLevelParams(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_expandWhereDecls(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__5; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); lean_object* l_Lean_MessageData_ofName(lean_object*); static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__5___lambda__4___closed__5; static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__5___closed__2; -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_declValToTerminationHint___spec__1___lambda__6___closed__1; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars_getFVars___closed__3; -static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__11; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__3(lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_FixPoint_getUsedFVarsMap___rarg(lean_object*); uint8_t l_Lean_Elab_Modifiers_isPartial(lean_object*); 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*); @@ -1236,11 +1247,13 @@ LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_MutualDef_ 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_object* l_Lean_Elab_Term_getLetRecsToLift___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__5___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Term_elabMutualDef_go___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___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* l_Lean_Expr_collectFVars(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_isTheorem___spec__1(lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Lean_RBNode_fold___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosures___spec__10(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_elabDeclAttrs___at_Lean_Elab_Command_elabMutualDef___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_declValToTerminationHint___spec__1___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_instInhabitedDefViewElabHeader___closed__5; size_t lean_usize_land(size_t, size_t); @@ -1253,9 +1266,9 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_Mutua LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3___closed__6; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars___spec__5(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__9; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_processDeriving___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars_collectUsed___spec__7(lean_object*, lean_object*, size_t, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__4; lean_object* l_Lean_profileitM___at_Lean_Meta_synthInstance_x3f___spec__6___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_MutualDef_0__Lean_Elab_Term_typeHasRecFun___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_FixPoint_isModified(lean_object*); @@ -1264,7 +1277,6 @@ LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_E uint8_t l_Lean_Expr_hasExprMVar(lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_elabMutualDef_go___spec__5___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_find___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_FixPoint_updateUsedVarsOf___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_cleanupOfNat___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_instantiateMVarsAtHeader(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1284,20 +1296,22 @@ return x_2; static lean_object* _init_l_Lean_Elab_instInhabitedDefViewElabHeader___closed__2() { _start: { -lean_object* x_1; uint8_t x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; +lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; uint8_t x_5; lean_object* x_6; lean_object* x_7; x_1 = lean_box(0); -x_2 = 0; +x_2 = lean_box(0); x_3 = 0; x_4 = 0; -x_5 = l_Lean_Elab_instInhabitedDefViewElabHeader___closed__1; -x_6 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_6, 0, x_1); -lean_ctor_set(x_6, 1, x_5); -lean_ctor_set_uint8(x_6, sizeof(void*)*2, x_2); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 1, x_3); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 2, x_4); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 3, x_3); -return x_6; +x_5 = 0; +x_6 = l_Lean_Elab_instInhabitedDefViewElabHeader___closed__1; +x_7 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_7, 0, x_2); +lean_ctor_set(x_7, 1, x_1); +lean_ctor_set(x_7, 2, x_6); +lean_ctor_set_uint8(x_7, sizeof(void*)*3, x_3); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 1, x_4); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 2, x_5); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 3, x_4); +return x_7; } } static lean_object* _init_l_Lean_Elab_instInhabitedDefViewElabHeader___closed__3() { @@ -1473,11 +1487,11 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check _start: { lean_object* x_11; uint8_t x_19; -x_19 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 1); +x_19 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 1); if (x_19 == 0) { uint8_t x_20; -x_20 = lean_ctor_get_uint8(x_2, sizeof(void*)*2 + 1); +x_20 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 1); if (x_20 == 0) { lean_object* x_21; lean_object* x_22; @@ -1496,7 +1510,7 @@ goto block_18; else { uint8_t x_24; -x_24 = lean_ctor_get_uint8(x_2, sizeof(void*)*2 + 1); +x_24 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 1); if (x_24 == 0) { lean_object* x_25; @@ -1560,11 +1574,11 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check _start: { lean_object* x_10; uint8_t x_18; -x_18 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 3); +x_18 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 3); if (x_18 == 0) { uint8_t x_19; -x_19 = lean_ctor_get_uint8(x_2, sizeof(void*)*2 + 3); +x_19 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 3); if (x_19 == 0) { lean_object* x_20; lean_object* x_21; @@ -1583,7 +1597,7 @@ goto block_17; else { uint8_t x_23; -x_23 = lean_ctor_get_uint8(x_2, sizeof(void*)*2 + 3); +x_23 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 3); if (x_23 == 0) { lean_object* x_24; @@ -2147,7 +2161,7 @@ return x_15; else { uint8_t x_16; -x_16 = lean_ctor_get_uint8(x_12, sizeof(void*)*2 + 3); +x_16 = lean_ctor_get_uint8(x_12, sizeof(void*)*3 + 3); if (x_16 == 0) { lean_object* x_17; lean_object* x_18; @@ -2205,7 +2219,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check lean_object* x_11; lean_object* x_12; uint8_t x_13; x_11 = lean_ctor_get(x_2, 0); x_12 = lean_ctor_get(x_11, 2); -x_13 = lean_ctor_get_uint8(x_12, sizeof(void*)*2 + 1); +x_13 = lean_ctor_get_uint8(x_12, sizeof(void*)*3 + 1); if (x_13 == 0) { lean_object* x_14; lean_object* x_15; @@ -2286,7 +2300,7 @@ else { lean_object* x_16; uint8_t x_17; x_16 = lean_ctor_get(x_11, 2); -x_17 = lean_ctor_get_uint8(x_16, sizeof(void*)*2 + 1); +x_17 = lean_ctor_get_uint8(x_16, sizeof(void*)*3 + 1); if (x_17 == 0) { lean_object* x_18; lean_object* x_19; @@ -2426,7 +2440,7 @@ else { lean_object* x_15; uint8_t x_16; x_15 = lean_ctor_get(x_10, 2); -x_16 = lean_ctor_get_uint8(x_15, sizeof(void*)*2 + 3); +x_16 = lean_ctor_get_uint8(x_15, sizeof(void*)*3 + 3); if (x_16 == 0) { lean_object* x_17; lean_object* x_18; @@ -8118,7 +8132,7 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Mutua lean_object* x_25; lean_object* x_26; lean_object* x_27; x_25 = lean_ctor_get(x_1, 2); lean_inc(x_25); -x_26 = lean_ctor_get(x_25, 1); +x_26 = lean_ctor_get(x_25, 2); lean_inc(x_26); lean_dec(x_25); lean_inc(x_23); @@ -21632,7 +21646,130 @@ return x_48; } } } -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +uint8_t x_11; lean_object* x_12; +x_11 = 1; +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_12 = l_Lean_Elab_Term_elabTermEnsuringType(x_1, x_2, x_11, x_11, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_12) == 0) +{ +lean_object* x_13; lean_object* x_14; uint8_t x_15; uint8_t x_16; lean_object* x_17; +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_12, 1); +lean_inc(x_14); +lean_dec(x_12); +x_15 = 1; +x_16 = 0; +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +x_17 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_15, x_16, x_4, x_5, x_6, x_7, x_8, x_9, x_14); +if (lean_obj_tag(x_17) == 0) +{ +lean_object* x_18; lean_object* x_19; +x_18 = lean_ctor_get(x_17, 1); +lean_inc(x_18); +lean_dec(x_17); +x_19 = l_Lean_Elab_Term_instantiateMVarsProfiling(x_13, x_6, x_7, x_8, x_9, x_18); +return x_19; +} +else +{ +uint8_t x_20; +lean_dec(x_13); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +x_20 = !lean_is_exclusive(x_17); +if (x_20 == 0) +{ +return x_17; +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_17, 0); +x_22 = lean_ctor_get(x_17, 1); +lean_inc(x_22); +lean_inc(x_21); +lean_dec(x_17); +x_23 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_23, 0, x_21); +lean_ctor_set(x_23, 1, x_22); +return x_23; +} +} +} +else +{ +uint8_t x_24; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_24 = !lean_is_exclusive(x_12); +if (x_24 == 0) +{ +return x_12; +} +else +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_12, 0); +x_26 = lean_ctor_get(x_12, 1); +lean_inc(x_26); +lean_inc(x_25); +lean_dec(x_12); +x_27 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +return x_27; +} +} +} +} +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("body", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__12___lambda__2___closed__5; +x_2 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__1; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; uint8_t x_12; lean_object* x_13; +x_11 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__2; +x_12 = 0; +lean_inc(x_2); +x_13 = l_Lean_Elab_Term_mkTermInfo(x_11, x_1, x_3, x_2, x_2, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { lean_object* x_10; @@ -21642,7 +21779,7 @@ lean_ctor_set(x_10, 1, x_9); return x_10; } } -static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__1() { +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__1() { _start: { lean_object* x_1; @@ -21650,7 +21787,7 @@ x_1 = l_Lean_Elab_Term_linter_unusedSectionVars; return x_1; } } -static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__2() { +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__2() { _start: { lean_object* x_1; @@ -21658,16 +21795,16 @@ x_1 = lean_mk_string_unchecked("automatically included section variable(s) unuse return x_1; } } -static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__3() { +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__2; +x_1 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__2; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__4() { +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__4() { _start: { lean_object* x_1; @@ -21675,16 +21812,16 @@ x_1 = lean_mk_string_unchecked("':\n ", 5, 5); return x_1; } } -static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__5() { +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__5() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__4; +x_1 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__4; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__6() { +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__6() { _start: { lean_object* x_1; @@ -21692,26 +21829,26 @@ x_1 = lean_mk_string_unchecked("\n ", 3, 3); return x_1; } } -static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__7() { +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__7() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__6; +x_1 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__6; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__8() { +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__8() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__7; +x_1 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__7; x_2 = l_Lean_MessageData_ofFormat(x_1); return x_2; } } -static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__9() { +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__9() { _start: { lean_object* x_1; @@ -21719,16 +21856,16 @@ x_1 = lean_mk_string_unchecked("\nconsider restructuring your `variable` declara return x_1; } } -static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__10() { +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__10() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__9; +x_1 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__9; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__11() { +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__11() { _start: { lean_object* x_1; @@ -21736,26 +21873,26 @@ x_1 = lean_mk_string_unchecked(" ", 1, 1); return x_1; } } -static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__12() { +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__12() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__11; +x_1 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__11; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__13() { +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__13() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__12; +x_1 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__12; x_2 = l_Lean_MessageData_ofFormat(x_1); return x_2; } } -static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__14() { +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__14() { _start: { lean_object* x_1; @@ -21763,16 +21900,16 @@ x_1 = lean_mk_string_unchecked(" in theorem ...", 15, 15); return x_1; } } -static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__15() { +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__15() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__14; +x_1 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__14; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19) { +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19) { _start: { lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; @@ -21798,119 +21935,101 @@ lean_dec(x_24); lean_dec(x_21); if (lean_obj_tag(x_26) == 0) { -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; uint8_t x_34; uint8_t x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; uint8_t x_41; uint8_t x_42; uint8_t x_43; uint8_t x_44; lean_object* x_45; uint8_t x_46; uint8_t x_47; lean_object* x_48; uint8_t x_49; lean_object* x_50; +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; uint8_t x_36; uint8_t x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; uint8_t x_43; uint8_t x_44; uint8_t x_45; uint8_t x_46; lean_object* x_47; uint8_t x_48; uint8_t x_49; lean_object* x_50; lean_object* x_51; x_27 = lean_ctor_get(x_26, 1); lean_inc(x_27); lean_dec(x_26); x_28 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_28, 0, x_12); x_29 = lean_box(0); -x_30 = lean_ctor_get(x_13, 0); -lean_inc(x_30); -x_31 = lean_ctor_get(x_13, 1); -lean_inc(x_31); -x_32 = lean_ctor_get(x_13, 2); +lean_inc(x_4); +x_30 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__1), 10, 3); +lean_closure_set(x_30, 0, x_4); +lean_closure_set(x_30, 1, x_28); +lean_closure_set(x_30, 2, x_29); +lean_inc(x_4); +x_31 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___boxed), 10, 2); +lean_closure_set(x_31, 0, x_4); +lean_closure_set(x_31, 1, x_29); +x_32 = lean_ctor_get(x_13, 0); lean_inc(x_32); -x_33 = lean_ctor_get_uint8(x_13, sizeof(void*)*9); -x_34 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 1); -x_35 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 2); -x_36 = lean_ctor_get(x_13, 3); -lean_inc(x_36); -x_37 = lean_ctor_get(x_13, 4); -lean_inc(x_37); -x_38 = lean_ctor_get(x_13, 5); +x_33 = lean_ctor_get(x_13, 1); +lean_inc(x_33); +x_34 = lean_ctor_get(x_13, 2); +lean_inc(x_34); +x_35 = lean_ctor_get_uint8(x_13, sizeof(void*)*9); +x_36 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 1); +x_37 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 2); +x_38 = lean_ctor_get(x_13, 3); lean_inc(x_38); -x_39 = lean_ctor_get(x_13, 6); +x_39 = lean_ctor_get(x_13, 4); lean_inc(x_39); -x_40 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 3); -x_41 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 4); -x_42 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 5); -x_43 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 6); -x_44 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 7); -x_45 = lean_ctor_get(x_13, 7); -lean_inc(x_45); -x_46 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 8); -x_47 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 9); -x_48 = lean_alloc_ctor(0, 9, 10); -lean_ctor_set(x_48, 0, x_30); -lean_ctor_set(x_48, 1, x_31); -lean_ctor_set(x_48, 2, x_32); -lean_ctor_set(x_48, 3, x_36); -lean_ctor_set(x_48, 4, x_37); -lean_ctor_set(x_48, 5, x_38); -lean_ctor_set(x_48, 6, x_39); -lean_ctor_set(x_48, 7, x_45); -lean_ctor_set(x_48, 8, x_4); -lean_ctor_set_uint8(x_48, sizeof(void*)*9, x_33); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 1, x_34); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 2, x_35); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 3, x_40); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 4, x_41); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 5, x_42); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 6, x_43); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 7, x_44); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 8, x_46); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 9, x_47); -x_49 = 1; +x_40 = lean_ctor_get(x_13, 5); +lean_inc(x_40); +x_41 = lean_ctor_get(x_13, 6); +lean_inc(x_41); +x_42 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 3); +x_43 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 4); +x_44 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 5); +x_45 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 6); +x_46 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 7); +x_47 = lean_ctor_get(x_13, 7); +lean_inc(x_47); +x_48 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 8); +x_49 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 9); +x_50 = lean_alloc_ctor(0, 9, 10); +lean_ctor_set(x_50, 0, x_32); +lean_ctor_set(x_50, 1, x_33); +lean_ctor_set(x_50, 2, x_34); +lean_ctor_set(x_50, 3, x_38); +lean_ctor_set(x_50, 4, x_39); +lean_ctor_set(x_50, 5, x_40); +lean_ctor_set(x_50, 6, x_41); +lean_ctor_set(x_50, 7, x_47); +lean_ctor_set(x_50, 8, x_5); +lean_ctor_set_uint8(x_50, sizeof(void*)*9, x_35); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 1, x_36); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 2, x_37); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 3, x_42); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 4, x_43); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 5, x_44); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 6, x_45); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 7, x_46); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 8, x_48); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 9, x_49); lean_inc(x_18); lean_inc(x_17); lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); -lean_inc(x_48); -x_50 = l_Lean_Elab_Term_elabTermEnsuringType(x_5, x_28, x_49, x_49, x_29, x_48, x_14, x_15, x_16, x_17, x_18, x_27); -if (lean_obj_tag(x_50) == 0) +x_51 = l_Lean_Elab_Term_withInfoContext_x27(x_4, x_30, x_31, x_50, x_14, x_15, x_16, x_17, x_18, x_27); +if (lean_obj_tag(x_51) == 0) { -lean_object* x_51; lean_object* x_52; uint8_t x_53; uint8_t x_54; lean_object* x_55; -x_51 = lean_ctor_get(x_50, 0); -lean_inc(x_51); -x_52 = lean_ctor_get(x_50, 1); +lean_object* x_52; lean_object* x_53; uint8_t x_54; uint8_t x_55; uint8_t x_56; lean_object* x_57; +x_52 = lean_ctor_get(x_51, 0); lean_inc(x_52); -lean_dec(x_50); -x_53 = 1; +x_53 = lean_ctor_get(x_51, 1); +lean_inc(x_53); +lean_dec(x_51); x_54 = 0; -lean_inc(x_18); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_15); -lean_inc(x_14); -x_55 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_53, x_54, x_48, x_14, x_15, x_16, x_17, x_18, x_52); -if (lean_obj_tag(x_55) == 0) -{ -lean_object* x_56; lean_object* x_57; -x_56 = lean_ctor_get(x_55, 1); -lean_inc(x_56); -lean_dec(x_55); -lean_inc(x_18); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_15); -x_57 = l_Lean_Elab_Term_instantiateMVarsProfiling(x_51, x_15, x_16, x_17, x_18, x_56); +x_55 = 1; +x_56 = 1; +x_57 = l_Lean_Meta_mkLambdaFVars(x_11, x_52, x_54, x_55, x_54, x_56, x_15, x_16, x_17, x_18, x_53); if (lean_obj_tag(x_57) == 0) { -lean_object* x_58; lean_object* x_59; uint8_t x_60; lean_object* x_61; -x_58 = lean_ctor_get(x_57, 0); -lean_inc(x_58); -x_59 = lean_ctor_get(x_57, 1); -lean_inc(x_59); -lean_dec(x_57); -x_60 = 1; -x_61 = l_Lean_Meta_mkLambdaFVars(x_11, x_58, x_54, x_49, x_54, x_60, x_15, x_16, x_17, x_18, x_59); -if (lean_obj_tag(x_61) == 0) -{ -uint8_t x_62; -x_62 = !lean_is_exclusive(x_61); -if (x_62 == 0) +uint8_t x_58; +x_58 = !lean_is_exclusive(x_57); +if (x_58 == 0) { -lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; uint8_t x_67; -x_63 = lean_ctor_get(x_61, 0); -x_64 = lean_ctor_get(x_61, 1); -x_65 = lean_ctor_get(x_17, 2); -lean_inc(x_65); -x_66 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__1; -x_67 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_65, x_66); -lean_dec(x_65); -if (x_67 == 0) +lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; +x_59 = lean_ctor_get(x_57, 0); +x_60 = lean_ctor_get(x_57, 1); +x_61 = lean_ctor_get(x_17, 2); +lean_inc(x_61); +x_62 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__1; +x_63 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_61, x_62); +lean_dec(x_61); +if (x_63 == 0) { lean_dec(x_18); lean_dec(x_17); @@ -21919,39 +22038,39 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -return x_61; +return x_57; } else { -uint8_t x_68; -x_68 = l_Lean_Expr_hasSorry(x_6); -if (x_68 == 0) +uint8_t x_64; +x_64 = l_Lean_Expr_hasSorry(x_6); +if (x_64 == 0) { -uint8_t x_69; -x_69 = l_Lean_Expr_hasSorry(x_63); -if (x_69 == 0) +uint8_t x_65; +x_65 = l_Lean_Expr_hasSorry(x_59); +if (x_65 == 0) { -lean_object* x_70; lean_object* x_71; -lean_free_object(x_61); -x_70 = lean_array_get_size(x_7); +lean_object* x_66; lean_object* x_67; +lean_free_object(x_57); +x_66 = lean_array_get_size(x_7); lean_inc(x_15); -x_71 = l_Array_filterMapM___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__3(x_8, x_7, x_6, x_63, x_7, x_22, x_70, x_13, x_14, x_15, x_16, x_17, x_18, x_64); -lean_dec(x_70); -if (lean_obj_tag(x_71) == 0) +x_67 = l_Array_filterMapM___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__3(x_8, x_7, x_6, x_59, x_7, x_22, x_66, x_13, x_14, x_15, x_16, x_17, x_18, x_60); +lean_dec(x_66); +if (lean_obj_tag(x_67) == 0) { -uint8_t x_72; -x_72 = !lean_is_exclusive(x_71); -if (x_72 == 0) +uint8_t x_68; +x_68 = !lean_is_exclusive(x_67); +if (x_68 == 0) { -lean_object* x_73; lean_object* x_74; lean_object* x_75; uint8_t x_76; -x_73 = lean_ctor_get(x_71, 0); -x_74 = lean_ctor_get(x_71, 1); -x_75 = lean_array_get_size(x_73); -x_76 = lean_nat_dec_lt(x_22, x_75); -lean_dec(x_75); -if (x_76 == 0) +lean_object* x_69; lean_object* x_70; lean_object* x_71; uint8_t x_72; +x_69 = lean_ctor_get(x_67, 0); +x_70 = lean_ctor_get(x_67, 1); +x_71 = lean_array_get_size(x_69); +x_72 = lean_nat_dec_lt(x_22, x_71); +lean_dec(x_71); +if (x_72 == 0) { -lean_dec(x_73); +lean_dec(x_69); lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -21959,86 +22078,86 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -lean_ctor_set(x_71, 0, x_63); -return x_71; +lean_ctor_set(x_67, 0, x_59); +return x_67; } else { -lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; uint8_t x_95; -lean_free_object(x_71); -x_77 = lean_ctor_get(x_9, 0); -x_78 = l_Lean_MessageData_ofName(x_10); -x_79 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__3; -x_80 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_80, 0, x_79); -lean_ctor_set(x_80, 1, x_78); -x_81 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__5; +lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; uint8_t x_91; +lean_free_object(x_67); +x_73 = lean_ctor_get(x_9, 0); +x_74 = l_Lean_MessageData_ofName(x_10); +x_75 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__3; +x_76 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_76, 0, x_75); +lean_ctor_set(x_76, 1, x_74); +x_77 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__5; +x_78 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_78, 0, x_76); +lean_ctor_set(x_78, 1, x_77); +x_79 = lean_array_to_list(x_69); +x_80 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__8; +lean_inc(x_79); +x_81 = l_Lean_MessageData_joinSep(x_79, x_80); x_82 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_82, 0, x_80); +lean_ctor_set(x_82, 0, x_78); lean_ctor_set(x_82, 1, x_81); -x_83 = lean_array_to_list(x_73); -x_84 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__8; -lean_inc(x_83); -x_85 = l_Lean_MessageData_joinSep(x_83, x_84); -x_86 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_86, 0, x_82); -lean_ctor_set(x_86, 1, x_85); -x_87 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__10; -x_88 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_88, 0, x_86); -lean_ctor_set(x_88, 1, x_87); -x_89 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__13; -x_90 = l_Lean_MessageData_joinSep(x_83, x_89); -x_91 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_91, 0, x_88); -lean_ctor_set(x_91, 1, x_90); -x_92 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__15; -x_93 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_93, 0, x_91); -lean_ctor_set(x_93, 1, x_92); -x_94 = l_Lean_Linter_logLint___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__5(x_66, x_77, x_93, x_13, x_14, x_15, x_16, x_17, x_18, x_74); +x_83 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__10; +x_84 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_84, 0, x_82); +lean_ctor_set(x_84, 1, x_83); +x_85 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__13; +x_86 = l_Lean_MessageData_joinSep(x_79, x_85); +x_87 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_87, 0, x_84); +lean_ctor_set(x_87, 1, x_86); +x_88 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__15; +x_89 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_89, 0, x_87); +lean_ctor_set(x_89, 1, x_88); +x_90 = l_Lean_Linter_logLint___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__5(x_62, x_73, x_89, x_13, x_14, x_15, x_16, x_17, x_18, x_70); lean_dec(x_18); lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); -x_95 = !lean_is_exclusive(x_94); -if (x_95 == 0) +x_91 = !lean_is_exclusive(x_90); +if (x_91 == 0) { -lean_object* x_96; -x_96 = lean_ctor_get(x_94, 0); -lean_dec(x_96); -lean_ctor_set(x_94, 0, x_63); -return x_94; +lean_object* x_92; +x_92 = lean_ctor_get(x_90, 0); +lean_dec(x_92); +lean_ctor_set(x_90, 0, x_59); +return x_90; } else { -lean_object* x_97; lean_object* x_98; -x_97 = lean_ctor_get(x_94, 1); -lean_inc(x_97); -lean_dec(x_94); -x_98 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_98, 0, x_63); -lean_ctor_set(x_98, 1, x_97); -return x_98; +lean_object* x_93; lean_object* x_94; +x_93 = lean_ctor_get(x_90, 1); +lean_inc(x_93); +lean_dec(x_90); +x_94 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_94, 0, x_59); +lean_ctor_set(x_94, 1, x_93); +return x_94; } } } else { -lean_object* x_99; lean_object* x_100; lean_object* x_101; uint8_t x_102; -x_99 = lean_ctor_get(x_71, 0); -x_100 = lean_ctor_get(x_71, 1); -lean_inc(x_100); -lean_inc(x_99); -lean_dec(x_71); -x_101 = lean_array_get_size(x_99); -x_102 = lean_nat_dec_lt(x_22, x_101); -lean_dec(x_101); -if (x_102 == 0) +lean_object* x_95; lean_object* x_96; lean_object* x_97; uint8_t x_98; +x_95 = lean_ctor_get(x_67, 0); +x_96 = lean_ctor_get(x_67, 1); +lean_inc(x_96); +lean_inc(x_95); +lean_dec(x_67); +x_97 = lean_array_get_size(x_95); +x_98 = lean_nat_dec_lt(x_22, x_97); +lean_dec(x_97); +if (x_98 == 0) { -lean_object* x_103; -lean_dec(x_99); +lean_object* x_99; +lean_dec(x_95); lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -22046,75 +22165,75 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -x_103 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_103, 0, x_63); -lean_ctor_set(x_103, 1, x_100); -return x_103; -} -else -{ -lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; -x_104 = lean_ctor_get(x_9, 0); -x_105 = l_Lean_MessageData_ofName(x_10); -x_106 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__3; -x_107 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_107, 0, x_106); -lean_ctor_set(x_107, 1, x_105); -x_108 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__5; +x_99 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_99, 0, x_59); +lean_ctor_set(x_99, 1, x_96); +return x_99; +} +else +{ +lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; +x_100 = lean_ctor_get(x_9, 0); +x_101 = l_Lean_MessageData_ofName(x_10); +x_102 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__3; +x_103 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_103, 0, x_102); +lean_ctor_set(x_103, 1, x_101); +x_104 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__5; +x_105 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_105, 0, x_103); +lean_ctor_set(x_105, 1, x_104); +x_106 = lean_array_to_list(x_95); +x_107 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__8; +lean_inc(x_106); +x_108 = l_Lean_MessageData_joinSep(x_106, x_107); x_109 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_109, 0, x_107); +lean_ctor_set(x_109, 0, x_105); lean_ctor_set(x_109, 1, x_108); -x_110 = lean_array_to_list(x_99); -x_111 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__8; -lean_inc(x_110); -x_112 = l_Lean_MessageData_joinSep(x_110, x_111); -x_113 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_113, 0, x_109); -lean_ctor_set(x_113, 1, x_112); -x_114 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__10; -x_115 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_115, 0, x_113); -lean_ctor_set(x_115, 1, x_114); -x_116 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__13; -x_117 = l_Lean_MessageData_joinSep(x_110, x_116); -x_118 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_118, 0, x_115); -lean_ctor_set(x_118, 1, x_117); -x_119 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__15; -x_120 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_120, 0, x_118); -lean_ctor_set(x_120, 1, x_119); -x_121 = l_Lean_Linter_logLint___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__5(x_66, x_104, x_120, x_13, x_14, x_15, x_16, x_17, x_18, x_100); +x_110 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__10; +x_111 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_111, 0, x_109); +lean_ctor_set(x_111, 1, x_110); +x_112 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__13; +x_113 = l_Lean_MessageData_joinSep(x_106, x_112); +x_114 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_114, 0, x_111); +lean_ctor_set(x_114, 1, x_113); +x_115 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__15; +x_116 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_116, 0, x_114); +lean_ctor_set(x_116, 1, x_115); +x_117 = l_Lean_Linter_logLint___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__5(x_62, x_100, x_116, x_13, x_14, x_15, x_16, x_17, x_18, x_96); lean_dec(x_18); lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); -x_122 = lean_ctor_get(x_121, 1); -lean_inc(x_122); -if (lean_is_exclusive(x_121)) { - lean_ctor_release(x_121, 0); - lean_ctor_release(x_121, 1); - x_123 = x_121; +x_118 = lean_ctor_get(x_117, 1); +lean_inc(x_118); +if (lean_is_exclusive(x_117)) { + lean_ctor_release(x_117, 0); + lean_ctor_release(x_117, 1); + x_119 = x_117; } else { - lean_dec_ref(x_121); - x_123 = lean_box(0); + lean_dec_ref(x_117); + x_119 = lean_box(0); } -if (lean_is_scalar(x_123)) { - x_124 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_119)) { + x_120 = lean_alloc_ctor(0, 2, 0); } else { - x_124 = x_123; + x_120 = x_119; } -lean_ctor_set(x_124, 0, x_63); -lean_ctor_set(x_124, 1, x_122); -return x_124; +lean_ctor_set(x_120, 0, x_59); +lean_ctor_set(x_120, 1, x_118); +return x_120; } } } else { -uint8_t x_125; -lean_dec(x_63); +uint8_t x_121; +lean_dec(x_59); lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -22122,23 +22241,23 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -x_125 = !lean_is_exclusive(x_71); -if (x_125 == 0) +x_121 = !lean_is_exclusive(x_67); +if (x_121 == 0) { -return x_71; +return x_67; } else { -lean_object* x_126; lean_object* x_127; lean_object* x_128; -x_126 = lean_ctor_get(x_71, 0); -x_127 = lean_ctor_get(x_71, 1); -lean_inc(x_127); -lean_inc(x_126); -lean_dec(x_71); -x_128 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_128, 0, x_126); -lean_ctor_set(x_128, 1, x_127); -return x_128; +lean_object* x_122; lean_object* x_123; lean_object* x_124; +x_122 = lean_ctor_get(x_67, 0); +x_123 = lean_ctor_get(x_67, 1); +lean_inc(x_123); +lean_inc(x_122); +lean_dec(x_67); +x_124 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_124, 0, x_122); +lean_ctor_set(x_124, 1, x_123); +return x_124; } } } @@ -22151,7 +22270,7 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -return x_61; +return x_57; } } else @@ -22163,26 +22282,26 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -return x_61; +return x_57; } } } else { -lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; uint8_t x_133; -x_129 = lean_ctor_get(x_61, 0); -x_130 = lean_ctor_get(x_61, 1); -lean_inc(x_130); -lean_inc(x_129); -lean_dec(x_61); -x_131 = lean_ctor_get(x_17, 2); -lean_inc(x_131); -x_132 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__1; -x_133 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_131, x_132); -lean_dec(x_131); -if (x_133 == 0) +lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; uint8_t x_129; +x_125 = lean_ctor_get(x_57, 0); +x_126 = lean_ctor_get(x_57, 1); +lean_inc(x_126); +lean_inc(x_125); +lean_dec(x_57); +x_127 = lean_ctor_get(x_17, 2); +lean_inc(x_127); +x_128 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__1; +x_129 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_127, x_128); +lean_dec(x_127); +if (x_129 == 0) { -lean_object* x_134; +lean_object* x_130; lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -22190,48 +22309,48 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -x_134 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_134, 0, x_129); -lean_ctor_set(x_134, 1, x_130); -return x_134; +x_130 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_130, 0, x_125); +lean_ctor_set(x_130, 1, x_126); +return x_130; } else { -uint8_t x_135; -x_135 = l_Lean_Expr_hasSorry(x_6); -if (x_135 == 0) +uint8_t x_131; +x_131 = l_Lean_Expr_hasSorry(x_6); +if (x_131 == 0) { -uint8_t x_136; -x_136 = l_Lean_Expr_hasSorry(x_129); -if (x_136 == 0) +uint8_t x_132; +x_132 = l_Lean_Expr_hasSorry(x_125); +if (x_132 == 0) { -lean_object* x_137; lean_object* x_138; -x_137 = lean_array_get_size(x_7); +lean_object* x_133; lean_object* x_134; +x_133 = lean_array_get_size(x_7); lean_inc(x_15); -x_138 = l_Array_filterMapM___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__3(x_8, x_7, x_6, x_129, x_7, x_22, x_137, x_13, x_14, x_15, x_16, x_17, x_18, x_130); -lean_dec(x_137); -if (lean_obj_tag(x_138) == 0) +x_134 = l_Array_filterMapM___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__3(x_8, x_7, x_6, x_125, x_7, x_22, x_133, x_13, x_14, x_15, x_16, x_17, x_18, x_126); +lean_dec(x_133); +if (lean_obj_tag(x_134) == 0) { -lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; uint8_t x_143; -x_139 = lean_ctor_get(x_138, 0); -lean_inc(x_139); -x_140 = lean_ctor_get(x_138, 1); -lean_inc(x_140); -if (lean_is_exclusive(x_138)) { - lean_ctor_release(x_138, 0); - lean_ctor_release(x_138, 1); - x_141 = x_138; +lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; uint8_t x_139; +x_135 = lean_ctor_get(x_134, 0); +lean_inc(x_135); +x_136 = lean_ctor_get(x_134, 1); +lean_inc(x_136); +if (lean_is_exclusive(x_134)) { + lean_ctor_release(x_134, 0); + lean_ctor_release(x_134, 1); + x_137 = x_134; } else { - lean_dec_ref(x_138); - x_141 = lean_box(0); + lean_dec_ref(x_134); + x_137 = lean_box(0); } -x_142 = lean_array_get_size(x_139); -x_143 = lean_nat_dec_lt(x_22, x_142); -lean_dec(x_142); -if (x_143 == 0) +x_138 = lean_array_get_size(x_135); +x_139 = lean_nat_dec_lt(x_22, x_138); +lean_dec(x_138); +if (x_139 == 0) { -lean_object* x_144; -lean_dec(x_139); +lean_object* x_140; +lean_dec(x_135); lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -22239,79 +22358,79 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -if (lean_is_scalar(x_141)) { - x_144 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_137)) { + x_140 = lean_alloc_ctor(0, 2, 0); } else { - x_144 = x_141; + x_140 = x_137; } -lean_ctor_set(x_144, 0, x_129); -lean_ctor_set(x_144, 1, x_140); -return x_144; +lean_ctor_set(x_140, 0, x_125); +lean_ctor_set(x_140, 1, x_136); +return x_140; } else { -lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; -lean_dec(x_141); -x_145 = lean_ctor_get(x_9, 0); -x_146 = l_Lean_MessageData_ofName(x_10); -x_147 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__3; -x_148 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_148, 0, x_147); -lean_ctor_set(x_148, 1, x_146); -x_149 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__5; +lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; +lean_dec(x_137); +x_141 = lean_ctor_get(x_9, 0); +x_142 = l_Lean_MessageData_ofName(x_10); +x_143 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__3; +x_144 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_144, 0, x_143); +lean_ctor_set(x_144, 1, x_142); +x_145 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__5; +x_146 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_146, 0, x_144); +lean_ctor_set(x_146, 1, x_145); +x_147 = lean_array_to_list(x_135); +x_148 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__8; +lean_inc(x_147); +x_149 = l_Lean_MessageData_joinSep(x_147, x_148); x_150 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_150, 0, x_148); +lean_ctor_set(x_150, 0, x_146); lean_ctor_set(x_150, 1, x_149); -x_151 = lean_array_to_list(x_139); -x_152 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__8; -lean_inc(x_151); -x_153 = l_Lean_MessageData_joinSep(x_151, x_152); -x_154 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_154, 0, x_150); -lean_ctor_set(x_154, 1, x_153); -x_155 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__10; -x_156 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_156, 0, x_154); -lean_ctor_set(x_156, 1, x_155); -x_157 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__13; -x_158 = l_Lean_MessageData_joinSep(x_151, x_157); -x_159 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_159, 0, x_156); -lean_ctor_set(x_159, 1, x_158); -x_160 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__15; -x_161 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_161, 0, x_159); -lean_ctor_set(x_161, 1, x_160); -x_162 = l_Lean_Linter_logLint___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__5(x_132, x_145, x_161, x_13, x_14, x_15, x_16, x_17, x_18, x_140); +x_151 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__10; +x_152 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_152, 0, x_150); +lean_ctor_set(x_152, 1, x_151); +x_153 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__13; +x_154 = l_Lean_MessageData_joinSep(x_147, x_153); +x_155 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_155, 0, x_152); +lean_ctor_set(x_155, 1, x_154); +x_156 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__15; +x_157 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_157, 0, x_155); +lean_ctor_set(x_157, 1, x_156); +x_158 = l_Lean_Linter_logLint___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__5(x_128, x_141, x_157, x_13, x_14, x_15, x_16, x_17, x_18, x_136); lean_dec(x_18); lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); -x_163 = lean_ctor_get(x_162, 1); -lean_inc(x_163); -if (lean_is_exclusive(x_162)) { - lean_ctor_release(x_162, 0); - lean_ctor_release(x_162, 1); - x_164 = x_162; +x_159 = lean_ctor_get(x_158, 1); +lean_inc(x_159); +if (lean_is_exclusive(x_158)) { + lean_ctor_release(x_158, 0); + lean_ctor_release(x_158, 1); + x_160 = x_158; } else { - lean_dec_ref(x_162); - x_164 = lean_box(0); + lean_dec_ref(x_158); + x_160 = lean_box(0); } -if (lean_is_scalar(x_164)) { - x_165 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_160)) { + x_161 = lean_alloc_ctor(0, 2, 0); } else { - x_165 = x_164; + x_161 = x_160; } -lean_ctor_set(x_165, 0, x_129); -lean_ctor_set(x_165, 1, x_163); -return x_165; +lean_ctor_set(x_161, 0, x_125); +lean_ctor_set(x_161, 1, x_159); +return x_161; } } else { -lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; -lean_dec(x_129); +lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; +lean_dec(x_125); lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -22319,47 +22438,31 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -x_166 = lean_ctor_get(x_138, 0); -lean_inc(x_166); -x_167 = lean_ctor_get(x_138, 1); -lean_inc(x_167); -if (lean_is_exclusive(x_138)) { - lean_ctor_release(x_138, 0); - lean_ctor_release(x_138, 1); - x_168 = x_138; +x_162 = lean_ctor_get(x_134, 0); +lean_inc(x_162); +x_163 = lean_ctor_get(x_134, 1); +lean_inc(x_163); +if (lean_is_exclusive(x_134)) { + lean_ctor_release(x_134, 0); + lean_ctor_release(x_134, 1); + x_164 = x_134; } else { - lean_dec_ref(x_138); - x_168 = lean_box(0); + lean_dec_ref(x_134); + x_164 = lean_box(0); } -if (lean_is_scalar(x_168)) { - x_169 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_164)) { + x_165 = lean_alloc_ctor(1, 2, 0); } else { - x_169 = x_168; -} -lean_ctor_set(x_169, 0, x_166); -lean_ctor_set(x_169, 1, x_167); -return x_169; -} + x_165 = x_164; } -else -{ -lean_object* x_170; -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_10); -x_170 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_170, 0, x_129); -lean_ctor_set(x_170, 1, x_130); -return x_170; +lean_ctor_set(x_165, 0, x_162); +lean_ctor_set(x_165, 1, x_163); +return x_165; } } else { -lean_object* x_171; +lean_object* x_166; lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -22367,17 +22470,15 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -x_171 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_171, 0, x_129); -lean_ctor_set(x_171, 1, x_130); -return x_171; -} -} +x_166 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_166, 0, x_125); +lean_ctor_set(x_166, 1, x_126); +return x_166; } } else { -uint8_t x_172; +lean_object* x_167; lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -22385,93 +22486,47 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -x_172 = !lean_is_exclusive(x_61); -if (x_172 == 0) -{ -return x_61; +x_167 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_167, 0, x_125); +lean_ctor_set(x_167, 1, x_126); +return x_167; } -else -{ -lean_object* x_173; lean_object* x_174; lean_object* x_175; -x_173 = lean_ctor_get(x_61, 0); -x_174 = lean_ctor_get(x_61, 1); -lean_inc(x_174); -lean_inc(x_173); -lean_dec(x_61); -x_175 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_175, 0, x_173); -lean_ctor_set(x_175, 1, x_174); -return x_175; } } } else { -uint8_t x_176; +uint8_t x_168; lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); -lean_dec(x_11); lean_dec(x_10); -x_176 = !lean_is_exclusive(x_57); -if (x_176 == 0) +x_168 = !lean_is_exclusive(x_57); +if (x_168 == 0) { return x_57; } else { -lean_object* x_177; lean_object* x_178; lean_object* x_179; -x_177 = lean_ctor_get(x_57, 0); -x_178 = lean_ctor_get(x_57, 1); -lean_inc(x_178); -lean_inc(x_177); +lean_object* x_169; lean_object* x_170; lean_object* x_171; +x_169 = lean_ctor_get(x_57, 0); +x_170 = lean_ctor_get(x_57, 1); +lean_inc(x_170); +lean_inc(x_169); lean_dec(x_57); -x_179 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_179, 0, x_177); -lean_ctor_set(x_179, 1, x_178); -return x_179; -} -} -} -else -{ -uint8_t x_180; -lean_dec(x_51); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_11); -lean_dec(x_10); -x_180 = !lean_is_exclusive(x_55); -if (x_180 == 0) -{ -return x_55; -} -else -{ -lean_object* x_181; lean_object* x_182; lean_object* x_183; -x_181 = lean_ctor_get(x_55, 0); -x_182 = lean_ctor_get(x_55, 1); -lean_inc(x_182); -lean_inc(x_181); -lean_dec(x_55); -x_183 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_183, 0, x_181); -lean_ctor_set(x_183, 1, x_182); -return x_183; +x_171 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_171, 0, x_169); +lean_ctor_set(x_171, 1, x_170); +return x_171; } } } else { -uint8_t x_184; -lean_dec(x_48); +uint8_t x_172; lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -22480,29 +22535,29 @@ lean_dec(x_14); lean_dec(x_13); lean_dec(x_11); lean_dec(x_10); -x_184 = !lean_is_exclusive(x_50); -if (x_184 == 0) +x_172 = !lean_is_exclusive(x_51); +if (x_172 == 0) { -return x_50; +return x_51; } else { -lean_object* x_185; lean_object* x_186; lean_object* x_187; -x_185 = lean_ctor_get(x_50, 0); -x_186 = lean_ctor_get(x_50, 1); -lean_inc(x_186); -lean_inc(x_185); -lean_dec(x_50); -x_187 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_187, 0, x_185); -lean_ctor_set(x_187, 1, x_186); -return x_187; +lean_object* x_173; lean_object* x_174; lean_object* x_175; +x_173 = lean_ctor_get(x_51, 0); +x_174 = lean_ctor_get(x_51, 1); +lean_inc(x_174); +lean_inc(x_173); +lean_dec(x_51); +x_175 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_175, 0, x_173); +lean_ctor_set(x_175, 1, x_174); +return x_175; } } } else { -uint8_t x_188; +uint8_t x_176; lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -22514,28 +22569,28 @@ lean_dec(x_11); lean_dec(x_10); lean_dec(x_5); lean_dec(x_4); -x_188 = !lean_is_exclusive(x_26); -if (x_188 == 0) +x_176 = !lean_is_exclusive(x_26); +if (x_176 == 0) { return x_26; } else { -lean_object* x_189; lean_object* x_190; lean_object* x_191; -x_189 = lean_ctor_get(x_26, 0); -x_190 = lean_ctor_get(x_26, 1); -lean_inc(x_190); -lean_inc(x_189); +lean_object* x_177; lean_object* x_178; lean_object* x_179; +x_177 = lean_ctor_get(x_26, 0); +x_178 = lean_ctor_get(x_26, 1); +lean_inc(x_178); +lean_inc(x_177); lean_dec(x_26); -x_191 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_191, 0, x_189); -lean_ctor_set(x_191, 1, x_190); -return x_191; +x_179 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_179, 0, x_177); +lean_ctor_set(x_179, 1, x_178); +return x_179; } } } } -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19) { +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19) { _start: { lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; @@ -22561,119 +22616,101 @@ lean_dec(x_24); lean_dec(x_21); if (lean_obj_tag(x_26) == 0) { -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; uint8_t x_34; uint8_t x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; uint8_t x_41; uint8_t x_42; uint8_t x_43; uint8_t x_44; lean_object* x_45; uint8_t x_46; uint8_t x_47; lean_object* x_48; uint8_t x_49; lean_object* x_50; +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; uint8_t x_36; uint8_t x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; uint8_t x_43; uint8_t x_44; uint8_t x_45; uint8_t x_46; lean_object* x_47; uint8_t x_48; uint8_t x_49; lean_object* x_50; lean_object* x_51; x_27 = lean_ctor_get(x_26, 1); lean_inc(x_27); lean_dec(x_26); x_28 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_28, 0, x_12); x_29 = lean_box(0); -x_30 = lean_ctor_get(x_13, 0); -lean_inc(x_30); -x_31 = lean_ctor_get(x_13, 1); -lean_inc(x_31); -x_32 = lean_ctor_get(x_13, 2); +lean_inc(x_4); +x_30 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__1), 10, 3); +lean_closure_set(x_30, 0, x_4); +lean_closure_set(x_30, 1, x_28); +lean_closure_set(x_30, 2, x_29); +lean_inc(x_4); +x_31 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___boxed), 10, 2); +lean_closure_set(x_31, 0, x_4); +lean_closure_set(x_31, 1, x_29); +x_32 = lean_ctor_get(x_13, 0); lean_inc(x_32); -x_33 = lean_ctor_get_uint8(x_13, sizeof(void*)*9); -x_34 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 1); -x_35 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 2); -x_36 = lean_ctor_get(x_13, 3); -lean_inc(x_36); -x_37 = lean_ctor_get(x_13, 4); -lean_inc(x_37); -x_38 = lean_ctor_get(x_13, 5); +x_33 = lean_ctor_get(x_13, 1); +lean_inc(x_33); +x_34 = lean_ctor_get(x_13, 2); +lean_inc(x_34); +x_35 = lean_ctor_get_uint8(x_13, sizeof(void*)*9); +x_36 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 1); +x_37 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 2); +x_38 = lean_ctor_get(x_13, 3); lean_inc(x_38); -x_39 = lean_ctor_get(x_13, 6); +x_39 = lean_ctor_get(x_13, 4); lean_inc(x_39); -x_40 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 3); -x_41 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 4); -x_42 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 5); -x_43 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 6); -x_44 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 7); -x_45 = lean_ctor_get(x_13, 7); -lean_inc(x_45); -x_46 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 8); -x_47 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 9); -x_48 = lean_alloc_ctor(0, 9, 10); -lean_ctor_set(x_48, 0, x_30); -lean_ctor_set(x_48, 1, x_31); -lean_ctor_set(x_48, 2, x_32); -lean_ctor_set(x_48, 3, x_36); -lean_ctor_set(x_48, 4, x_37); -lean_ctor_set(x_48, 5, x_38); -lean_ctor_set(x_48, 6, x_39); -lean_ctor_set(x_48, 7, x_45); -lean_ctor_set(x_48, 8, x_4); -lean_ctor_set_uint8(x_48, sizeof(void*)*9, x_33); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 1, x_34); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 2, x_35); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 3, x_40); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 4, x_41); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 5, x_42); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 6, x_43); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 7, x_44); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 8, x_46); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 9, x_47); -x_49 = 1; +x_40 = lean_ctor_get(x_13, 5); +lean_inc(x_40); +x_41 = lean_ctor_get(x_13, 6); +lean_inc(x_41); +x_42 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 3); +x_43 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 4); +x_44 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 5); +x_45 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 6); +x_46 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 7); +x_47 = lean_ctor_get(x_13, 7); +lean_inc(x_47); +x_48 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 8); +x_49 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 9); +x_50 = lean_alloc_ctor(0, 9, 10); +lean_ctor_set(x_50, 0, x_32); +lean_ctor_set(x_50, 1, x_33); +lean_ctor_set(x_50, 2, x_34); +lean_ctor_set(x_50, 3, x_38); +lean_ctor_set(x_50, 4, x_39); +lean_ctor_set(x_50, 5, x_40); +lean_ctor_set(x_50, 6, x_41); +lean_ctor_set(x_50, 7, x_47); +lean_ctor_set(x_50, 8, x_5); +lean_ctor_set_uint8(x_50, sizeof(void*)*9, x_35); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 1, x_36); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 2, x_37); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 3, x_42); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 4, x_43); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 5, x_44); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 6, x_45); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 7, x_46); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 8, x_48); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 9, x_49); lean_inc(x_18); lean_inc(x_17); lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); -lean_inc(x_48); -x_50 = l_Lean_Elab_Term_elabTermEnsuringType(x_5, x_28, x_49, x_49, x_29, x_48, x_14, x_15, x_16, x_17, x_18, x_27); -if (lean_obj_tag(x_50) == 0) +x_51 = l_Lean_Elab_Term_withInfoContext_x27(x_4, x_30, x_31, x_50, x_14, x_15, x_16, x_17, x_18, x_27); +if (lean_obj_tag(x_51) == 0) { -lean_object* x_51; lean_object* x_52; uint8_t x_53; uint8_t x_54; lean_object* x_55; -x_51 = lean_ctor_get(x_50, 0); -lean_inc(x_51); -x_52 = lean_ctor_get(x_50, 1); +lean_object* x_52; lean_object* x_53; uint8_t x_54; uint8_t x_55; uint8_t x_56; lean_object* x_57; +x_52 = lean_ctor_get(x_51, 0); lean_inc(x_52); -lean_dec(x_50); -x_53 = 1; +x_53 = lean_ctor_get(x_51, 1); +lean_inc(x_53); +lean_dec(x_51); x_54 = 0; -lean_inc(x_18); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_15); -lean_inc(x_14); -x_55 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_53, x_54, x_48, x_14, x_15, x_16, x_17, x_18, x_52); -if (lean_obj_tag(x_55) == 0) -{ -lean_object* x_56; lean_object* x_57; -x_56 = lean_ctor_get(x_55, 1); -lean_inc(x_56); -lean_dec(x_55); -lean_inc(x_18); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_15); -x_57 = l_Lean_Elab_Term_instantiateMVarsProfiling(x_51, x_15, x_16, x_17, x_18, x_56); +x_55 = 1; +x_56 = 1; +x_57 = l_Lean_Meta_mkLambdaFVars(x_11, x_52, x_54, x_55, x_54, x_56, x_15, x_16, x_17, x_18, x_53); if (lean_obj_tag(x_57) == 0) { -lean_object* x_58; lean_object* x_59; uint8_t x_60; lean_object* x_61; -x_58 = lean_ctor_get(x_57, 0); -lean_inc(x_58); -x_59 = lean_ctor_get(x_57, 1); -lean_inc(x_59); -lean_dec(x_57); -x_60 = 1; -x_61 = l_Lean_Meta_mkLambdaFVars(x_11, x_58, x_54, x_49, x_54, x_60, x_15, x_16, x_17, x_18, x_59); -if (lean_obj_tag(x_61) == 0) -{ -uint8_t x_62; -x_62 = !lean_is_exclusive(x_61); -if (x_62 == 0) +uint8_t x_58; +x_58 = !lean_is_exclusive(x_57); +if (x_58 == 0) { -lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; uint8_t x_67; -x_63 = lean_ctor_get(x_61, 0); -x_64 = lean_ctor_get(x_61, 1); -x_65 = lean_ctor_get(x_17, 2); -lean_inc(x_65); -x_66 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__1; -x_67 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_65, x_66); -lean_dec(x_65); -if (x_67 == 0) +lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; +x_59 = lean_ctor_get(x_57, 0); +x_60 = lean_ctor_get(x_57, 1); +x_61 = lean_ctor_get(x_17, 2); +lean_inc(x_61); +x_62 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__1; +x_63 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_61, x_62); +lean_dec(x_61); +if (x_63 == 0) { lean_dec(x_18); lean_dec(x_17); @@ -22682,39 +22719,39 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -return x_61; +return x_57; } else { -uint8_t x_68; -x_68 = l_Lean_Expr_hasSorry(x_6); -if (x_68 == 0) +uint8_t x_64; +x_64 = l_Lean_Expr_hasSorry(x_6); +if (x_64 == 0) { -uint8_t x_69; -x_69 = l_Lean_Expr_hasSorry(x_63); -if (x_69 == 0) +uint8_t x_65; +x_65 = l_Lean_Expr_hasSorry(x_59); +if (x_65 == 0) { -lean_object* x_70; lean_object* x_71; -lean_free_object(x_61); -x_70 = lean_array_get_size(x_7); +lean_object* x_66; lean_object* x_67; +lean_free_object(x_57); +x_66 = lean_array_get_size(x_7); lean_inc(x_15); -x_71 = l_Array_filterMapM___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__8(x_8, x_7, x_6, x_63, x_7, x_22, x_70, x_13, x_14, x_15, x_16, x_17, x_18, x_64); -lean_dec(x_70); -if (lean_obj_tag(x_71) == 0) +x_67 = l_Array_filterMapM___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__8(x_8, x_7, x_6, x_59, x_7, x_22, x_66, x_13, x_14, x_15, x_16, x_17, x_18, x_60); +lean_dec(x_66); +if (lean_obj_tag(x_67) == 0) { -uint8_t x_72; -x_72 = !lean_is_exclusive(x_71); -if (x_72 == 0) +uint8_t x_68; +x_68 = !lean_is_exclusive(x_67); +if (x_68 == 0) { -lean_object* x_73; lean_object* x_74; lean_object* x_75; uint8_t x_76; -x_73 = lean_ctor_get(x_71, 0); -x_74 = lean_ctor_get(x_71, 1); -x_75 = lean_array_get_size(x_73); -x_76 = lean_nat_dec_lt(x_22, x_75); -lean_dec(x_75); -if (x_76 == 0) +lean_object* x_69; lean_object* x_70; lean_object* x_71; uint8_t x_72; +x_69 = lean_ctor_get(x_67, 0); +x_70 = lean_ctor_get(x_67, 1); +x_71 = lean_array_get_size(x_69); +x_72 = lean_nat_dec_lt(x_22, x_71); +lean_dec(x_71); +if (x_72 == 0) { -lean_dec(x_73); +lean_dec(x_69); lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -22722,86 +22759,86 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -lean_ctor_set(x_71, 0, x_63); -return x_71; +lean_ctor_set(x_67, 0, x_59); +return x_67; } else { -lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; uint8_t x_95; -lean_free_object(x_71); -x_77 = lean_ctor_get(x_9, 0); -x_78 = l_Lean_MessageData_ofName(x_10); -x_79 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__3; -x_80 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_80, 0, x_79); -lean_ctor_set(x_80, 1, x_78); -x_81 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__5; +lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; uint8_t x_91; +lean_free_object(x_67); +x_73 = lean_ctor_get(x_9, 0); +x_74 = l_Lean_MessageData_ofName(x_10); +x_75 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__3; +x_76 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_76, 0, x_75); +lean_ctor_set(x_76, 1, x_74); +x_77 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__5; +x_78 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_78, 0, x_76); +lean_ctor_set(x_78, 1, x_77); +x_79 = lean_array_to_list(x_69); +x_80 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__8; +lean_inc(x_79); +x_81 = l_Lean_MessageData_joinSep(x_79, x_80); x_82 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_82, 0, x_80); +lean_ctor_set(x_82, 0, x_78); lean_ctor_set(x_82, 1, x_81); -x_83 = lean_array_to_list(x_73); -x_84 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__8; -lean_inc(x_83); -x_85 = l_Lean_MessageData_joinSep(x_83, x_84); -x_86 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_86, 0, x_82); -lean_ctor_set(x_86, 1, x_85); -x_87 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__10; -x_88 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_88, 0, x_86); -lean_ctor_set(x_88, 1, x_87); -x_89 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__13; -x_90 = l_Lean_MessageData_joinSep(x_83, x_89); -x_91 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_91, 0, x_88); -lean_ctor_set(x_91, 1, x_90); -x_92 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__15; -x_93 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_93, 0, x_91); -lean_ctor_set(x_93, 1, x_92); -x_94 = l_Lean_Linter_logLint___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__5(x_66, x_77, x_93, x_13, x_14, x_15, x_16, x_17, x_18, x_74); +x_83 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__10; +x_84 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_84, 0, x_82); +lean_ctor_set(x_84, 1, x_83); +x_85 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__13; +x_86 = l_Lean_MessageData_joinSep(x_79, x_85); +x_87 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_87, 0, x_84); +lean_ctor_set(x_87, 1, x_86); +x_88 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__15; +x_89 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_89, 0, x_87); +lean_ctor_set(x_89, 1, x_88); +x_90 = l_Lean_Linter_logLint___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__5(x_62, x_73, x_89, x_13, x_14, x_15, x_16, x_17, x_18, x_70); lean_dec(x_18); lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); -x_95 = !lean_is_exclusive(x_94); -if (x_95 == 0) +x_91 = !lean_is_exclusive(x_90); +if (x_91 == 0) { -lean_object* x_96; -x_96 = lean_ctor_get(x_94, 0); -lean_dec(x_96); -lean_ctor_set(x_94, 0, x_63); -return x_94; +lean_object* x_92; +x_92 = lean_ctor_get(x_90, 0); +lean_dec(x_92); +lean_ctor_set(x_90, 0, x_59); +return x_90; } else { -lean_object* x_97; lean_object* x_98; -x_97 = lean_ctor_get(x_94, 1); -lean_inc(x_97); -lean_dec(x_94); -x_98 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_98, 0, x_63); -lean_ctor_set(x_98, 1, x_97); -return x_98; +lean_object* x_93; lean_object* x_94; +x_93 = lean_ctor_get(x_90, 1); +lean_inc(x_93); +lean_dec(x_90); +x_94 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_94, 0, x_59); +lean_ctor_set(x_94, 1, x_93); +return x_94; } } } else { -lean_object* x_99; lean_object* x_100; lean_object* x_101; uint8_t x_102; -x_99 = lean_ctor_get(x_71, 0); -x_100 = lean_ctor_get(x_71, 1); -lean_inc(x_100); -lean_inc(x_99); -lean_dec(x_71); -x_101 = lean_array_get_size(x_99); -x_102 = lean_nat_dec_lt(x_22, x_101); -lean_dec(x_101); -if (x_102 == 0) +lean_object* x_95; lean_object* x_96; lean_object* x_97; uint8_t x_98; +x_95 = lean_ctor_get(x_67, 0); +x_96 = lean_ctor_get(x_67, 1); +lean_inc(x_96); +lean_inc(x_95); +lean_dec(x_67); +x_97 = lean_array_get_size(x_95); +x_98 = lean_nat_dec_lt(x_22, x_97); +lean_dec(x_97); +if (x_98 == 0) { -lean_object* x_103; -lean_dec(x_99); +lean_object* x_99; +lean_dec(x_95); lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -22809,75 +22846,75 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -x_103 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_103, 0, x_63); -lean_ctor_set(x_103, 1, x_100); -return x_103; -} -else -{ -lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; -x_104 = lean_ctor_get(x_9, 0); -x_105 = l_Lean_MessageData_ofName(x_10); -x_106 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__3; -x_107 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_107, 0, x_106); -lean_ctor_set(x_107, 1, x_105); -x_108 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__5; +x_99 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_99, 0, x_59); +lean_ctor_set(x_99, 1, x_96); +return x_99; +} +else +{ +lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; +x_100 = lean_ctor_get(x_9, 0); +x_101 = l_Lean_MessageData_ofName(x_10); +x_102 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__3; +x_103 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_103, 0, x_102); +lean_ctor_set(x_103, 1, x_101); +x_104 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__5; +x_105 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_105, 0, x_103); +lean_ctor_set(x_105, 1, x_104); +x_106 = lean_array_to_list(x_95); +x_107 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__8; +lean_inc(x_106); +x_108 = l_Lean_MessageData_joinSep(x_106, x_107); x_109 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_109, 0, x_107); +lean_ctor_set(x_109, 0, x_105); lean_ctor_set(x_109, 1, x_108); -x_110 = lean_array_to_list(x_99); -x_111 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__8; -lean_inc(x_110); -x_112 = l_Lean_MessageData_joinSep(x_110, x_111); -x_113 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_113, 0, x_109); -lean_ctor_set(x_113, 1, x_112); -x_114 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__10; -x_115 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_115, 0, x_113); -lean_ctor_set(x_115, 1, x_114); -x_116 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__13; -x_117 = l_Lean_MessageData_joinSep(x_110, x_116); -x_118 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_118, 0, x_115); -lean_ctor_set(x_118, 1, x_117); -x_119 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__15; -x_120 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_120, 0, x_118); -lean_ctor_set(x_120, 1, x_119); -x_121 = l_Lean_Linter_logLint___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__5(x_66, x_104, x_120, x_13, x_14, x_15, x_16, x_17, x_18, x_100); +x_110 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__10; +x_111 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_111, 0, x_109); +lean_ctor_set(x_111, 1, x_110); +x_112 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__13; +x_113 = l_Lean_MessageData_joinSep(x_106, x_112); +x_114 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_114, 0, x_111); +lean_ctor_set(x_114, 1, x_113); +x_115 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__15; +x_116 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_116, 0, x_114); +lean_ctor_set(x_116, 1, x_115); +x_117 = l_Lean_Linter_logLint___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__5(x_62, x_100, x_116, x_13, x_14, x_15, x_16, x_17, x_18, x_96); lean_dec(x_18); lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); -x_122 = lean_ctor_get(x_121, 1); -lean_inc(x_122); -if (lean_is_exclusive(x_121)) { - lean_ctor_release(x_121, 0); - lean_ctor_release(x_121, 1); - x_123 = x_121; +x_118 = lean_ctor_get(x_117, 1); +lean_inc(x_118); +if (lean_is_exclusive(x_117)) { + lean_ctor_release(x_117, 0); + lean_ctor_release(x_117, 1); + x_119 = x_117; } else { - lean_dec_ref(x_121); - x_123 = lean_box(0); + lean_dec_ref(x_117); + x_119 = lean_box(0); } -if (lean_is_scalar(x_123)) { - x_124 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_119)) { + x_120 = lean_alloc_ctor(0, 2, 0); } else { - x_124 = x_123; + x_120 = x_119; } -lean_ctor_set(x_124, 0, x_63); -lean_ctor_set(x_124, 1, x_122); -return x_124; +lean_ctor_set(x_120, 0, x_59); +lean_ctor_set(x_120, 1, x_118); +return x_120; } } } else { -uint8_t x_125; -lean_dec(x_63); +uint8_t x_121; +lean_dec(x_59); lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -22885,23 +22922,23 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -x_125 = !lean_is_exclusive(x_71); -if (x_125 == 0) +x_121 = !lean_is_exclusive(x_67); +if (x_121 == 0) { -return x_71; +return x_67; } else { -lean_object* x_126; lean_object* x_127; lean_object* x_128; -x_126 = lean_ctor_get(x_71, 0); -x_127 = lean_ctor_get(x_71, 1); -lean_inc(x_127); -lean_inc(x_126); -lean_dec(x_71); -x_128 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_128, 0, x_126); -lean_ctor_set(x_128, 1, x_127); -return x_128; +lean_object* x_122; lean_object* x_123; lean_object* x_124; +x_122 = lean_ctor_get(x_67, 0); +x_123 = lean_ctor_get(x_67, 1); +lean_inc(x_123); +lean_inc(x_122); +lean_dec(x_67); +x_124 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_124, 0, x_122); +lean_ctor_set(x_124, 1, x_123); +return x_124; } } } @@ -22914,7 +22951,7 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -return x_61; +return x_57; } } else @@ -22926,26 +22963,26 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -return x_61; +return x_57; } } } else { -lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; uint8_t x_133; -x_129 = lean_ctor_get(x_61, 0); -x_130 = lean_ctor_get(x_61, 1); -lean_inc(x_130); -lean_inc(x_129); -lean_dec(x_61); -x_131 = lean_ctor_get(x_17, 2); -lean_inc(x_131); -x_132 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__1; -x_133 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_131, x_132); -lean_dec(x_131); -if (x_133 == 0) +lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; uint8_t x_129; +x_125 = lean_ctor_get(x_57, 0); +x_126 = lean_ctor_get(x_57, 1); +lean_inc(x_126); +lean_inc(x_125); +lean_dec(x_57); +x_127 = lean_ctor_get(x_17, 2); +lean_inc(x_127); +x_128 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__1; +x_129 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_127, x_128); +lean_dec(x_127); +if (x_129 == 0) { -lean_object* x_134; +lean_object* x_130; lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -22953,48 +22990,48 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -x_134 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_134, 0, x_129); -lean_ctor_set(x_134, 1, x_130); -return x_134; +x_130 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_130, 0, x_125); +lean_ctor_set(x_130, 1, x_126); +return x_130; } else { -uint8_t x_135; -x_135 = l_Lean_Expr_hasSorry(x_6); -if (x_135 == 0) +uint8_t x_131; +x_131 = l_Lean_Expr_hasSorry(x_6); +if (x_131 == 0) { -uint8_t x_136; -x_136 = l_Lean_Expr_hasSorry(x_129); -if (x_136 == 0) +uint8_t x_132; +x_132 = l_Lean_Expr_hasSorry(x_125); +if (x_132 == 0) { -lean_object* x_137; lean_object* x_138; -x_137 = lean_array_get_size(x_7); +lean_object* x_133; lean_object* x_134; +x_133 = lean_array_get_size(x_7); lean_inc(x_15); -x_138 = l_Array_filterMapM___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__8(x_8, x_7, x_6, x_129, x_7, x_22, x_137, x_13, x_14, x_15, x_16, x_17, x_18, x_130); -lean_dec(x_137); -if (lean_obj_tag(x_138) == 0) +x_134 = l_Array_filterMapM___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__8(x_8, x_7, x_6, x_125, x_7, x_22, x_133, x_13, x_14, x_15, x_16, x_17, x_18, x_126); +lean_dec(x_133); +if (lean_obj_tag(x_134) == 0) { -lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; uint8_t x_143; -x_139 = lean_ctor_get(x_138, 0); -lean_inc(x_139); -x_140 = lean_ctor_get(x_138, 1); -lean_inc(x_140); -if (lean_is_exclusive(x_138)) { - lean_ctor_release(x_138, 0); - lean_ctor_release(x_138, 1); - x_141 = x_138; +lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; uint8_t x_139; +x_135 = lean_ctor_get(x_134, 0); +lean_inc(x_135); +x_136 = lean_ctor_get(x_134, 1); +lean_inc(x_136); +if (lean_is_exclusive(x_134)) { + lean_ctor_release(x_134, 0); + lean_ctor_release(x_134, 1); + x_137 = x_134; } else { - lean_dec_ref(x_138); - x_141 = lean_box(0); + lean_dec_ref(x_134); + x_137 = lean_box(0); } -x_142 = lean_array_get_size(x_139); -x_143 = lean_nat_dec_lt(x_22, x_142); -lean_dec(x_142); -if (x_143 == 0) +x_138 = lean_array_get_size(x_135); +x_139 = lean_nat_dec_lt(x_22, x_138); +lean_dec(x_138); +if (x_139 == 0) { -lean_object* x_144; -lean_dec(x_139); +lean_object* x_140; +lean_dec(x_135); lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -23002,79 +23039,79 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -if (lean_is_scalar(x_141)) { - x_144 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_137)) { + x_140 = lean_alloc_ctor(0, 2, 0); } else { - x_144 = x_141; + x_140 = x_137; } -lean_ctor_set(x_144, 0, x_129); -lean_ctor_set(x_144, 1, x_140); -return x_144; +lean_ctor_set(x_140, 0, x_125); +lean_ctor_set(x_140, 1, x_136); +return x_140; } else { -lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; -lean_dec(x_141); -x_145 = lean_ctor_get(x_9, 0); -x_146 = l_Lean_MessageData_ofName(x_10); -x_147 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__3; -x_148 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_148, 0, x_147); -lean_ctor_set(x_148, 1, x_146); -x_149 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__5; +lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; +lean_dec(x_137); +x_141 = lean_ctor_get(x_9, 0); +x_142 = l_Lean_MessageData_ofName(x_10); +x_143 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__3; +x_144 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_144, 0, x_143); +lean_ctor_set(x_144, 1, x_142); +x_145 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__5; +x_146 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_146, 0, x_144); +lean_ctor_set(x_146, 1, x_145); +x_147 = lean_array_to_list(x_135); +x_148 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__8; +lean_inc(x_147); +x_149 = l_Lean_MessageData_joinSep(x_147, x_148); x_150 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_150, 0, x_148); +lean_ctor_set(x_150, 0, x_146); lean_ctor_set(x_150, 1, x_149); -x_151 = lean_array_to_list(x_139); -x_152 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__8; -lean_inc(x_151); -x_153 = l_Lean_MessageData_joinSep(x_151, x_152); -x_154 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_154, 0, x_150); -lean_ctor_set(x_154, 1, x_153); -x_155 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__10; -x_156 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_156, 0, x_154); -lean_ctor_set(x_156, 1, x_155); -x_157 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__13; -x_158 = l_Lean_MessageData_joinSep(x_151, x_157); -x_159 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_159, 0, x_156); -lean_ctor_set(x_159, 1, x_158); -x_160 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__15; -x_161 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_161, 0, x_159); -lean_ctor_set(x_161, 1, x_160); -x_162 = l_Lean_Linter_logLint___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__5(x_132, x_145, x_161, x_13, x_14, x_15, x_16, x_17, x_18, x_140); +x_151 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__10; +x_152 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_152, 0, x_150); +lean_ctor_set(x_152, 1, x_151); +x_153 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__13; +x_154 = l_Lean_MessageData_joinSep(x_147, x_153); +x_155 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_155, 0, x_152); +lean_ctor_set(x_155, 1, x_154); +x_156 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__15; +x_157 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_157, 0, x_155); +lean_ctor_set(x_157, 1, x_156); +x_158 = l_Lean_Linter_logLint___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__5(x_128, x_141, x_157, x_13, x_14, x_15, x_16, x_17, x_18, x_136); lean_dec(x_18); lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); -x_163 = lean_ctor_get(x_162, 1); -lean_inc(x_163); -if (lean_is_exclusive(x_162)) { - lean_ctor_release(x_162, 0); - lean_ctor_release(x_162, 1); - x_164 = x_162; +x_159 = lean_ctor_get(x_158, 1); +lean_inc(x_159); +if (lean_is_exclusive(x_158)) { + lean_ctor_release(x_158, 0); + lean_ctor_release(x_158, 1); + x_160 = x_158; } else { - lean_dec_ref(x_162); - x_164 = lean_box(0); + lean_dec_ref(x_158); + x_160 = lean_box(0); } -if (lean_is_scalar(x_164)) { - x_165 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_160)) { + x_161 = lean_alloc_ctor(0, 2, 0); } else { - x_165 = x_164; + x_161 = x_160; } -lean_ctor_set(x_165, 0, x_129); -lean_ctor_set(x_165, 1, x_163); -return x_165; +lean_ctor_set(x_161, 0, x_125); +lean_ctor_set(x_161, 1, x_159); +return x_161; } } else { -lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; -lean_dec(x_129); +lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; +lean_dec(x_125); lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -23082,31 +23119,31 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -x_166 = lean_ctor_get(x_138, 0); -lean_inc(x_166); -x_167 = lean_ctor_get(x_138, 1); -lean_inc(x_167); -if (lean_is_exclusive(x_138)) { - lean_ctor_release(x_138, 0); - lean_ctor_release(x_138, 1); - x_168 = x_138; +x_162 = lean_ctor_get(x_134, 0); +lean_inc(x_162); +x_163 = lean_ctor_get(x_134, 1); +lean_inc(x_163); +if (lean_is_exclusive(x_134)) { + lean_ctor_release(x_134, 0); + lean_ctor_release(x_134, 1); + x_164 = x_134; } else { - lean_dec_ref(x_138); - x_168 = lean_box(0); + lean_dec_ref(x_134); + x_164 = lean_box(0); } -if (lean_is_scalar(x_168)) { - x_169 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_164)) { + x_165 = lean_alloc_ctor(1, 2, 0); } else { - x_169 = x_168; + x_165 = x_164; } -lean_ctor_set(x_169, 0, x_166); -lean_ctor_set(x_169, 1, x_167); -return x_169; +lean_ctor_set(x_165, 0, x_162); +lean_ctor_set(x_165, 1, x_163); +return x_165; } } else { -lean_object* x_170; +lean_object* x_166; lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -23114,15 +23151,15 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -x_170 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_170, 0, x_129); -lean_ctor_set(x_170, 1, x_130); -return x_170; +x_166 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_166, 0, x_125); +lean_ctor_set(x_166, 1, x_126); +return x_166; } } else { -lean_object* x_171; +lean_object* x_167; lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -23130,17 +23167,17 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -x_171 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_171, 0, x_129); -lean_ctor_set(x_171, 1, x_130); -return x_171; +x_167 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_167, 0, x_125); +lean_ctor_set(x_167, 1, x_126); +return x_167; } } } } else { -uint8_t x_172; +uint8_t x_168; lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -23148,93 +23185,29 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -x_172 = !lean_is_exclusive(x_61); -if (x_172 == 0) -{ -return x_61; -} -else -{ -lean_object* x_173; lean_object* x_174; lean_object* x_175; -x_173 = lean_ctor_get(x_61, 0); -x_174 = lean_ctor_get(x_61, 1); -lean_inc(x_174); -lean_inc(x_173); -lean_dec(x_61); -x_175 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_175, 0, x_173); -lean_ctor_set(x_175, 1, x_174); -return x_175; -} -} -} -else -{ -uint8_t x_176; -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_11); -lean_dec(x_10); -x_176 = !lean_is_exclusive(x_57); -if (x_176 == 0) +x_168 = !lean_is_exclusive(x_57); +if (x_168 == 0) { return x_57; } else { -lean_object* x_177; lean_object* x_178; lean_object* x_179; -x_177 = lean_ctor_get(x_57, 0); -x_178 = lean_ctor_get(x_57, 1); -lean_inc(x_178); -lean_inc(x_177); +lean_object* x_169; lean_object* x_170; lean_object* x_171; +x_169 = lean_ctor_get(x_57, 0); +x_170 = lean_ctor_get(x_57, 1); +lean_inc(x_170); +lean_inc(x_169); lean_dec(x_57); -x_179 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_179, 0, x_177); -lean_ctor_set(x_179, 1, x_178); -return x_179; -} -} -} -else -{ -uint8_t x_180; -lean_dec(x_51); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_11); -lean_dec(x_10); -x_180 = !lean_is_exclusive(x_55); -if (x_180 == 0) -{ -return x_55; -} -else -{ -lean_object* x_181; lean_object* x_182; lean_object* x_183; -x_181 = lean_ctor_get(x_55, 0); -x_182 = lean_ctor_get(x_55, 1); -lean_inc(x_182); -lean_inc(x_181); -lean_dec(x_55); -x_183 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_183, 0, x_181); -lean_ctor_set(x_183, 1, x_182); -return x_183; +x_171 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_171, 0, x_169); +lean_ctor_set(x_171, 1, x_170); +return x_171; } } } else { -uint8_t x_184; -lean_dec(x_48); +uint8_t x_172; lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -23243,29 +23216,29 @@ lean_dec(x_14); lean_dec(x_13); lean_dec(x_11); lean_dec(x_10); -x_184 = !lean_is_exclusive(x_50); -if (x_184 == 0) +x_172 = !lean_is_exclusive(x_51); +if (x_172 == 0) { -return x_50; +return x_51; } else { -lean_object* x_185; lean_object* x_186; lean_object* x_187; -x_185 = lean_ctor_get(x_50, 0); -x_186 = lean_ctor_get(x_50, 1); -lean_inc(x_186); -lean_inc(x_185); -lean_dec(x_50); -x_187 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_187, 0, x_185); -lean_ctor_set(x_187, 1, x_186); -return x_187; +lean_object* x_173; lean_object* x_174; lean_object* x_175; +x_173 = lean_ctor_get(x_51, 0); +x_174 = lean_ctor_get(x_51, 1); +lean_inc(x_174); +lean_inc(x_173); +lean_dec(x_51); +x_175 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_175, 0, x_173); +lean_ctor_set(x_175, 1, x_174); +return x_175; } } } else { -uint8_t x_188; +uint8_t x_176; lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -23277,28 +23250,28 @@ lean_dec(x_11); lean_dec(x_10); lean_dec(x_5); lean_dec(x_4); -x_188 = !lean_is_exclusive(x_26); -if (x_188 == 0) +x_176 = !lean_is_exclusive(x_26); +if (x_176 == 0) { return x_26; } else { -lean_object* x_189; lean_object* x_190; lean_object* x_191; -x_189 = lean_ctor_get(x_26, 0); -x_190 = lean_ctor_get(x_26, 1); -lean_inc(x_190); -lean_inc(x_189); +lean_object* x_177; lean_object* x_178; lean_object* x_179; +x_177 = lean_ctor_get(x_26, 0); +x_178 = lean_ctor_get(x_26, 1); +lean_inc(x_178); +lean_inc(x_177); lean_dec(x_26); -x_191 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_191, 0, x_189); -lean_ctor_set(x_191, 1, x_190); -return x_191; +x_179 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_179, 0, x_177); +lean_ctor_set(x_179, 1, x_178); +return x_179; } } } } -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; lean_object* x_21; @@ -23310,7 +23283,7 @@ lean_inc(x_17); x_18 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_18, 0, x_17); lean_inc(x_16); -x_19 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__3___boxed), 19, 10); +x_19 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5___boxed), 19, 10); lean_closure_set(x_19, 0, x_1); lean_closure_set(x_19, 1, x_2); lean_closure_set(x_19, 2, x_17); @@ -23326,7 +23299,7 @@ x_21 = l_Lean_Meta_forallBoundedTelescope___at_Lean_Elab_Term_addAutoBoundImplic return x_21; } } -static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5___closed__1() { +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__7___closed__1() { _start: { lean_object* x_1; @@ -23334,7 +23307,7 @@ x_1 = l_Lean_Elab_Term_deprecated_oldSectionVars; return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { lean_object* x_16; @@ -23364,7 +23337,7 @@ goto block_27; else { lean_object* x_32; uint8_t x_33; -x_32 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5___closed__1; +x_32 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__7___closed__1; x_33 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_28, x_32); lean_dec(x_28); if (x_33 == 0) @@ -23372,11 +23345,11 @@ if (x_33 == 0) lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_inc(x_5); lean_inc(x_3); -x_34 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4), 15, 7); +x_34 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__6), 15, 7); lean_closure_set(x_34, 0, x_2); lean_closure_set(x_34, 1, x_3); -lean_closure_set(x_34, 2, x_4); -lean_closure_set(x_34, 3, x_17); +lean_closure_set(x_34, 2, x_17); +lean_closure_set(x_34, 3, x_4); lean_closure_set(x_34, 4, x_5); lean_closure_set(x_34, 5, x_6); lean_closure_set(x_34, 6, x_7); @@ -23411,12 +23384,12 @@ x_22 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_22, 0, x_21); x_23 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___closed__1; lean_inc(x_20); -x_24 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___boxed), 19, 10); +x_24 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___boxed), 19, 10); lean_closure_set(x_24, 0, x_2); lean_closure_set(x_24, 1, x_3); lean_closure_set(x_24, 2, x_21); -lean_closure_set(x_24, 3, x_4); -lean_closure_set(x_24, 4, x_17); +lean_closure_set(x_24, 3, x_17); +lean_closure_set(x_24, 4, x_4); lean_closure_set(x_24, 5, x_20); lean_closure_set(x_24, 6, x_23); lean_closure_set(x_24, 7, x_5); @@ -23463,7 +23436,7 @@ return x_43; } } } -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; uint8_t x_12; @@ -23698,7 +23671,7 @@ lean_inc(x_18); x_19 = lean_ctor_get(x_6, 2); lean_inc(x_19); lean_inc(x_7); -x_20 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5___boxed), 15, 8); +x_20 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__7___boxed), 15, 8); lean_closure_set(x_20, 0, x_8); lean_closure_set(x_20, 1, x_6); lean_closure_set(x_20, 2, x_3); @@ -23721,7 +23694,7 @@ x_24 = lean_ctor_get(x_10, 8); lean_dec(x_24); lean_ctor_set(x_10, 8, x_9); x_25 = lean_box(0); -x_26 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__6(x_18, x_22, x_10, x_11, x_12, x_13, x_25, x_15, x_16, x_17); +x_26 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__8(x_18, x_22, x_10, x_11, x_12, x_13, x_25, x_15, x_16, x_17); return x_26; } else @@ -23775,7 +23748,7 @@ lean_ctor_set_uint8(x_45, sizeof(void*)*9 + 7, x_41); lean_ctor_set_uint8(x_45, sizeof(void*)*9 + 8, x_43); lean_ctor_set_uint8(x_45, sizeof(void*)*9 + 9, x_44); x_46 = lean_box(0); -x_47 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__6(x_18, x_22, x_45, x_11, x_12, x_13, x_46, x_15, x_16, x_17); +x_47 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__8(x_18, x_22, x_45, x_11, x_12, x_13, x_46, x_15, x_16, x_17); return x_47; } } @@ -23893,7 +23866,7 @@ lean_inc(x_18); x_19 = lean_ctor_get(x_6, 2); lean_inc(x_19); lean_inc(x_7); -x_20 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5___boxed), 15, 8); +x_20 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__7___boxed), 15, 8); lean_closure_set(x_20, 0, x_8); lean_closure_set(x_20, 1, x_6); lean_closure_set(x_20, 2, x_3); @@ -23916,7 +23889,7 @@ x_24 = lean_ctor_get(x_10, 8); lean_dec(x_24); lean_ctor_set(x_10, 8, x_9); x_25 = lean_box(0); -x_26 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__6(x_18, x_22, x_10, x_11, x_12, x_13, x_25, x_15, x_16, x_17); +x_26 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__8(x_18, x_22, x_10, x_11, x_12, x_13, x_25, x_15, x_16, x_17); return x_26; } else @@ -23970,7 +23943,7 @@ lean_ctor_set_uint8(x_45, sizeof(void*)*9 + 7, x_41); lean_ctor_set_uint8(x_45, sizeof(void*)*9 + 8, x_43); lean_ctor_set_uint8(x_45, sizeof(void*)*9 + 9, x_44); x_46 = lean_box(0); -x_47 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__6(x_18, x_22, x_45, x_11, x_12, x_13, x_46, x_15, x_16, x_17); +x_47 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__8(x_18, x_22, x_45, x_11, x_12, x_13, x_46, x_15, x_16, x_17); return x_47; } } @@ -24574,7 +24547,7 @@ lean_inc(x_18); x_19 = lean_ctor_get(x_6, 2); lean_inc(x_19); lean_inc(x_7); -x_20 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5___boxed), 15, 8); +x_20 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__7___boxed), 15, 8); lean_closure_set(x_20, 0, x_8); lean_closure_set(x_20, 1, x_6); lean_closure_set(x_20, 2, x_3); @@ -24597,7 +24570,7 @@ x_24 = lean_ctor_get(x_10, 8); lean_dec(x_24); lean_ctor_set(x_10, 8, x_9); x_25 = lean_box(0); -x_26 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__6(x_18, x_22, x_10, x_11, x_12, x_13, x_25, x_15, x_16, x_17); +x_26 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__8(x_18, x_22, x_10, x_11, x_12, x_13, x_25, x_15, x_16, x_17); return x_26; } else @@ -24651,7 +24624,7 @@ lean_ctor_set_uint8(x_45, sizeof(void*)*9 + 7, x_41); lean_ctor_set_uint8(x_45, sizeof(void*)*9 + 8, x_43); lean_ctor_set_uint8(x_45, sizeof(void*)*9 + 9, x_44); x_46 = lean_box(0); -x_47 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__6(x_18, x_22, x_45, x_11, x_12, x_13, x_46, x_15, x_16, x_17); +x_47 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__8(x_18, x_22, x_45, x_11, x_12, x_13, x_46, x_15, x_16, x_17); return x_47; } } @@ -24769,7 +24742,7 @@ lean_inc(x_18); x_19 = lean_ctor_get(x_6, 2); lean_inc(x_19); lean_inc(x_7); -x_20 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5___boxed), 15, 8); +x_20 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__7___boxed), 15, 8); lean_closure_set(x_20, 0, x_8); lean_closure_set(x_20, 1, x_6); lean_closure_set(x_20, 2, x_3); @@ -24792,7 +24765,7 @@ x_24 = lean_ctor_get(x_10, 8); lean_dec(x_24); lean_ctor_set(x_10, 8, x_9); x_25 = lean_box(0); -x_26 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__6(x_18, x_22, x_10, x_11, x_12, x_13, x_25, x_15, x_16, x_17); +x_26 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__8(x_18, x_22, x_10, x_11, x_12, x_13, x_25, x_15, x_16, x_17); return x_26; } else @@ -24846,7 +24819,7 @@ lean_ctor_set_uint8(x_45, sizeof(void*)*9 + 7, x_41); lean_ctor_set_uint8(x_45, sizeof(void*)*9 + 8, x_43); lean_ctor_set_uint8(x_45, sizeof(void*)*9 + 9, x_44); x_46 = lean_box(0); -x_47 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__6(x_18, x_22, x_45, x_11, x_12, x_13, x_46, x_15, x_16, x_17); +x_47 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__8(x_18, x_22, x_45, x_11, x_12, x_13, x_46, x_15, x_16, x_17); return x_47; } } @@ -27155,11 +27128,25 @@ lean_dec(x_1); return x_15; } } -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { lean_object* x_10; -x_10 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_10 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -27170,7 +27157,7 @@ lean_dec(x_2); return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___boxed(lean_object** _args) { +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___boxed(lean_object** _args) { lean_object* x_1 = _args[0]; lean_object* x_2 = _args[1]; lean_object* x_3 = _args[2]; @@ -27193,7 +27180,7 @@ lean_object* x_19 = _args[18]; _start: { lean_object* x_20; -x_20 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19); +x_20 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -27204,7 +27191,7 @@ lean_dec(x_1); return x_20; } } -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__3___boxed(lean_object** _args) { +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5___boxed(lean_object** _args) { lean_object* x_1 = _args[0]; lean_object* x_2 = _args[1]; lean_object* x_3 = _args[2]; @@ -27227,7 +27214,7 @@ lean_object* x_19 = _args[18]; _start: { lean_object* x_20; -x_20 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19); +x_20 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -27238,20 +27225,20 @@ lean_dec(x_1); return x_20; } } -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { lean_object* x_16; -x_16 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +x_16 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__7(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); lean_dec(x_8); return x_16; } } -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; -x_11 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_7); return x_11; } @@ -37385,11 +37372,11 @@ x_14 = !lean_is_exclusive(x_1); if (x_14 == 0) { lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_15 = lean_ctor_get(x_1, 1); +x_15 = lean_ctor_get(x_1, 2); lean_dec(x_15); x_16 = lean_ctor_get(x_2, 2); lean_inc(x_16); -lean_ctor_set(x_1, 1, x_16); +lean_ctor_set(x_1, 2, x_16); x_17 = lean_ctor_get(x_2, 4); x_18 = lean_ctor_get(x_2, 10); lean_inc(x_18); @@ -37411,41 +37398,44 @@ return x_21; } else { -lean_object* x_22; uint8_t x_23; uint8_t x_24; uint8_t x_25; uint8_t x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +lean_object* x_22; lean_object* x_23; uint8_t x_24; uint8_t x_25; uint8_t x_26; uint8_t x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; x_22 = lean_ctor_get(x_1, 0); -x_23 = lean_ctor_get_uint8(x_1, sizeof(void*)*2); -x_24 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 1); -x_25 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 2); -x_26 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 3); +x_23 = lean_ctor_get(x_1, 1); +x_24 = lean_ctor_get_uint8(x_1, sizeof(void*)*3); +x_25 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 1); +x_26 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 2); +x_27 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 3); +lean_inc(x_23); lean_inc(x_22); lean_dec(x_1); -x_27 = lean_ctor_get(x_2, 2); -lean_inc(x_27); -x_28 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_28, 0, x_22); -lean_ctor_set(x_28, 1, x_27); -lean_ctor_set_uint8(x_28, sizeof(void*)*2, x_23); -lean_ctor_set_uint8(x_28, sizeof(void*)*2 + 1, x_24); -lean_ctor_set_uint8(x_28, sizeof(void*)*2 + 2, x_25); -lean_ctor_set_uint8(x_28, sizeof(void*)*2 + 3, x_26); -x_29 = lean_ctor_get(x_2, 4); -x_30 = lean_ctor_get(x_2, 10); +x_28 = lean_ctor_get(x_2, 2); +lean_inc(x_28); +x_29 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_29, 0, x_22); +lean_ctor_set(x_29, 1, x_23); +lean_ctor_set(x_29, 2, x_28); +lean_ctor_set_uint8(x_29, sizeof(void*)*3, x_24); +lean_ctor_set_uint8(x_29, sizeof(void*)*3 + 1, x_25); +lean_ctor_set_uint8(x_29, sizeof(void*)*3 + 2, x_26); +lean_ctor_set_uint8(x_29, sizeof(void*)*3 + 3, x_27); +x_30 = lean_ctor_get(x_2, 4); +x_31 = lean_ctor_get(x_2, 10); +lean_inc(x_31); lean_inc(x_30); -lean_inc(x_29); -x_31 = lean_alloc_ctor(0, 7, 1); -lean_ctor_set(x_31, 0, x_3); -lean_ctor_set(x_31, 1, x_13); -lean_ctor_set(x_31, 2, x_28); -lean_ctor_set(x_31, 3, x_29); -lean_ctor_set(x_31, 4, x_4); -lean_ctor_set(x_31, 5, x_5); -lean_ctor_set(x_31, 6, x_30); -lean_ctor_set_uint8(x_31, sizeof(void*)*7, x_7); -x_32 = lean_array_push(x_6, x_31); -x_33 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_33, 0, x_32); -lean_ctor_set(x_33, 1, x_12); -return x_33; +x_32 = lean_alloc_ctor(0, 7, 1); +lean_ctor_set(x_32, 0, x_3); +lean_ctor_set(x_32, 1, x_13); +lean_ctor_set(x_32, 2, x_29); +lean_ctor_set(x_32, 3, x_30); +lean_ctor_set(x_32, 4, x_4); +lean_ctor_set(x_32, 5, x_5); +lean_ctor_set(x_32, 6, x_31); +lean_ctor_set_uint8(x_32, sizeof(void*)*7, x_7); +x_33 = lean_array_push(x_6, x_32); +x_34 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_34, 0, x_33); +lean_ctor_set(x_34, 1, x_12); +return x_34; } } } @@ -37996,7 +37986,7 @@ lean_dec(x_5); x_7 = lean_ctor_get(x_6, 2); lean_inc(x_7); lean_dec(x_6); -x_8 = lean_ctor_get_uint8(x_7, sizeof(void*)*2 + 3); +x_8 = lean_ctor_get_uint8(x_7, sizeof(void*)*3 + 3); lean_dec(x_7); if (x_8 == 0) { @@ -38076,7 +38066,7 @@ lean_dec(x_5); x_7 = lean_ctor_get(x_6, 2); lean_inc(x_7); lean_dec(x_6); -x_8 = lean_ctor_get_uint8(x_7, sizeof(void*)*2 + 1); +x_8 = lean_ctor_get_uint8(x_7, sizeof(void*)*3 + 1); lean_dec(x_7); if (x_8 == 0) { @@ -38111,99 +38101,105 @@ x_4 = lean_unsigned_to_nat(0u); x_5 = lean_nat_dec_lt(x_4, x_3); if (x_5 == 0) { -uint8_t x_32; -x_32 = 0; -x_6 = x_32; -goto block_31; +uint8_t x_35; +x_35 = 0; +x_6 = x_35; +goto block_34; } else { -size_t x_33; size_t x_34; uint8_t x_35; -x_33 = 0; -x_34 = lean_usize_of_nat(x_3); -x_35 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_MutualClosure_getModifiersForLetRecs___spec__3(x_1, x_33, x_34); -x_6 = x_35; -goto block_31; +size_t x_36; size_t x_37; uint8_t x_38; +x_36 = 0; +x_37 = lean_usize_of_nat(x_3); +x_38 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_MutualClosure_getModifiersForLetRecs___spec__3(x_1, x_36, x_37); +x_6 = x_38; +goto block_34; } -block_31: +block_34: { lean_object* x_7; if (x_5 == 0) { -lean_object* x_21; -x_21 = lean_box(0); -x_7 = x_21; -goto block_20; +lean_object* x_23; +x_23 = lean_box(0); +x_7 = x_23; +goto block_22; } else { -size_t x_22; size_t x_23; uint8_t x_24; -x_22 = 0; -x_23 = lean_usize_of_nat(x_3); -x_24 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_MutualClosure_getModifiersForLetRecs___spec__2(x_1, x_22, x_23); -if (x_24 == 0) +size_t x_24; size_t x_25; uint8_t x_26; +x_24 = 0; +x_25 = lean_usize_of_nat(x_3); +x_26 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_MutualClosure_getModifiersForLetRecs___spec__2(x_1, x_24, x_25); +if (x_26 == 0) { -lean_object* x_25; -x_25 = lean_box(0); -x_7 = x_25; -goto block_20; +lean_object* x_27; +x_27 = lean_box(0); +x_7 = x_27; +goto block_22; } else { -uint8_t x_26; uint8_t x_27; uint8_t x_28; lean_object* x_29; lean_object* x_30; +uint8_t x_28; lean_object* x_29; uint8_t x_30; uint8_t x_31; lean_object* x_32; lean_object* x_33; lean_dec(x_3); -x_26 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_MutualClosure_getModifiersForLetRecs___spec__1(x_1, x_22, x_23); -x_27 = 0; -x_28 = 0; -x_29 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___closed__1; -x_30 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_30, 0, x_2); -lean_ctor_set(x_30, 1, x_29); -lean_ctor_set_uint8(x_30, sizeof(void*)*2, x_27); -lean_ctor_set_uint8(x_30, sizeof(void*)*2 + 1, x_6); -lean_ctor_set_uint8(x_30, sizeof(void*)*2 + 2, x_28); -lean_ctor_set_uint8(x_30, sizeof(void*)*2 + 3, x_26); -return x_30; +x_28 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_MutualClosure_getModifiersForLetRecs___spec__1(x_1, x_24, x_25); +x_29 = lean_box(0); +x_30 = 0; +x_31 = 0; +x_32 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___closed__1; +x_33 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_33, 0, x_29); +lean_ctor_set(x_33, 1, x_2); +lean_ctor_set(x_33, 2, x_32); +lean_ctor_set_uint8(x_33, sizeof(void*)*3, x_30); +lean_ctor_set_uint8(x_33, sizeof(void*)*3 + 1, x_6); +lean_ctor_set_uint8(x_33, sizeof(void*)*3 + 2, x_31); +lean_ctor_set_uint8(x_33, sizeof(void*)*3 + 3, x_28); +return x_33; } } -block_20: +block_22: { lean_dec(x_7); if (x_5 == 0) { -uint8_t x_8; uint8_t x_9; uint8_t x_10; lean_object* x_11; lean_object* x_12; +lean_object* x_8; uint8_t x_9; uint8_t x_10; uint8_t x_11; lean_object* x_12; lean_object* x_13; lean_dec(x_3); -x_8 = 0; -x_9 = 2; -x_10 = 0; -x_11 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___closed__1; -x_12 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_12, 0, x_2); -lean_ctor_set(x_12, 1, x_11); -lean_ctor_set_uint8(x_12, sizeof(void*)*2, x_8); -lean_ctor_set_uint8(x_12, sizeof(void*)*2 + 1, x_6); -lean_ctor_set_uint8(x_12, sizeof(void*)*2 + 2, x_9); -lean_ctor_set_uint8(x_12, sizeof(void*)*2 + 3, x_10); -return x_12; +x_8 = lean_box(0); +x_9 = 0; +x_10 = 2; +x_11 = 0; +x_12 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___closed__1; +x_13 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_13, 0, x_8); +lean_ctor_set(x_13, 1, x_2); +lean_ctor_set(x_13, 2, x_12); +lean_ctor_set_uint8(x_13, sizeof(void*)*3, x_9); +lean_ctor_set_uint8(x_13, sizeof(void*)*3 + 1, x_6); +lean_ctor_set_uint8(x_13, sizeof(void*)*3 + 2, x_10); +lean_ctor_set_uint8(x_13, sizeof(void*)*3 + 3, x_11); +return x_13; } else { -size_t x_13; size_t x_14; uint8_t x_15; uint8_t x_16; uint8_t x_17; lean_object* x_18; lean_object* x_19; -x_13 = 0; -x_14 = lean_usize_of_nat(x_3); +size_t x_14; size_t x_15; uint8_t x_16; lean_object* x_17; uint8_t x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; +x_14 = 0; +x_15 = lean_usize_of_nat(x_3); lean_dec(x_3); -x_15 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_MutualClosure_getModifiersForLetRecs___spec__1(x_1, x_13, x_14); -x_16 = 0; -x_17 = 2; -x_18 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___closed__1; -x_19 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_19, 0, x_2); -lean_ctor_set(x_19, 1, x_18); -lean_ctor_set_uint8(x_19, sizeof(void*)*2, x_16); -lean_ctor_set_uint8(x_19, sizeof(void*)*2 + 1, x_6); -lean_ctor_set_uint8(x_19, sizeof(void*)*2 + 2, x_17); -lean_ctor_set_uint8(x_19, sizeof(void*)*2 + 3, x_15); -return x_19; +x_16 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_MutualClosure_getModifiersForLetRecs___spec__1(x_1, x_14, x_15); +x_17 = lean_box(0); +x_18 = 0; +x_19 = 2; +x_20 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___closed__1; +x_21 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_21, 0, x_17); +lean_ctor_set(x_21, 1, x_2); +lean_ctor_set(x_21, 2, x_20); +lean_ctor_set_uint8(x_21, sizeof(void*)*3, x_18); +lean_ctor_set_uint8(x_21, sizeof(void*)*3 + 1, x_6); +lean_ctor_set_uint8(x_21, sizeof(void*)*3 + 2, x_19); +lean_ctor_set_uint8(x_21, sizeof(void*)*3 + 3, x_16); +return x_21; } } } @@ -42906,242 +42902,151 @@ return x_29; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Term_elabMutualDef_go___spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Term_elabMutualDef_go___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_9; uint8_t x_10; lean_object* x_11; lean_object* x_12; -x_9 = lean_ctor_get(x_6, 1); -lean_inc(x_9); -lean_dec(x_6); -x_10 = 0; -x_11 = l_Lean_Syntax_getPos_x3f(x_1, x_10); -x_12 = l_Lean_Syntax_getTailPos_x3f(x_1, x_10); -if (lean_obj_tag(x_11) == 0) +uint8_t x_9; lean_object* x_10; +x_9 = 0; +x_10 = l_Lean_Syntax_getRange_x3f(x_1, x_9); +if (lean_obj_tag(x_10) == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_unsigned_to_nat(0u); -lean_inc(x_9); -x_14 = l_Lean_FileMap_toPosition(x_9, x_13); -lean_inc(x_14); -x_15 = l_Lean_FileMap_leanPosToLspPos(x_9, x_14); -if (lean_obj_tag(x_12) == 0) +lean_object* x_11; lean_object* x_12; +lean_dec(x_6); +x_11 = lean_box(0); +x_12 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_11); +lean_ctor_set(x_12, 1, x_8); +return x_12; +} +else { -uint8_t x_16; -lean_dec(x_9); -x_16 = !lean_is_exclusive(x_15); -if (x_16 == 0) +uint8_t x_13; +x_13 = !lean_is_exclusive(x_10); +if (x_13 == 0) { -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_15, 1); -x_18 = lean_ctor_get(x_15, 0); +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_14 = lean_ctor_get(x_10, 0); +x_15 = lean_ctor_get(x_6, 1); +lean_inc(x_15); +lean_dec(x_6); +x_16 = lean_ctor_get(x_14, 0); +lean_inc(x_16); +lean_inc(x_15); +x_17 = l_Lean_FileMap_toPosition(x_15, x_16); +lean_dec(x_16); +x_18 = lean_ctor_get(x_14, 1); +lean_inc(x_18); +lean_dec(x_14); +lean_inc(x_15); +x_19 = l_Lean_FileMap_toPosition(x_15, x_18); lean_dec(x_18); lean_inc(x_17); -lean_inc(x_14); -x_19 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_19, 0, x_14); -lean_ctor_set(x_19, 1, x_17); -lean_ctor_set(x_19, 2, x_14); -lean_ctor_set(x_19, 3, x_17); -lean_ctor_set(x_15, 1, x_8); -lean_ctor_set(x_15, 0, x_19); -return x_15; -} -else +x_20 = l_Lean_FileMap_leanPosToLspPos(x_15, x_17); +x_21 = !lean_is_exclusive(x_20); +if (x_21 == 0) { -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_15, 1); -lean_inc(x_20); +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_22 = lean_ctor_get(x_20, 1); +x_23 = lean_ctor_get(x_20, 0); +lean_dec(x_23); +lean_inc(x_19); +x_24 = l_Lean_FileMap_leanPosToLspPos(x_15, x_19); lean_dec(x_15); -lean_inc(x_20); -lean_inc(x_14); -x_21 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_21, 0, x_14); -lean_ctor_set(x_21, 1, x_20); -lean_ctor_set(x_21, 2, x_14); -lean_ctor_set(x_21, 3, x_20); -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_21); -lean_ctor_set(x_22, 1, x_8); -return x_22; -} +x_25 = lean_ctor_get(x_24, 1); +lean_inc(x_25); +lean_dec(x_24); +x_26 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_26, 0, x_17); +lean_ctor_set(x_26, 1, x_22); +lean_ctor_set(x_26, 2, x_19); +lean_ctor_set(x_26, 3, x_25); +lean_ctor_set(x_10, 0, x_26); +lean_ctor_set(x_20, 1, x_8); +lean_ctor_set(x_20, 0, x_10); +return x_20; } else { -uint8_t x_23; -x_23 = !lean_is_exclusive(x_15); -if (x_23 == 0) -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_24 = lean_ctor_get(x_15, 1); -x_25 = lean_ctor_get(x_15, 0); -lean_dec(x_25); -x_26 = lean_ctor_get(x_12, 0); -lean_inc(x_26); -lean_dec(x_12); -lean_inc(x_9); -x_27 = l_Lean_FileMap_toPosition(x_9, x_26); -lean_dec(x_26); +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_27 = lean_ctor_get(x_20, 1); lean_inc(x_27); -x_28 = l_Lean_FileMap_leanPosToLspPos(x_9, x_27); -lean_dec(x_9); +lean_dec(x_20); +lean_inc(x_19); +x_28 = l_Lean_FileMap_leanPosToLspPos(x_15, x_19); +lean_dec(x_15); x_29 = lean_ctor_get(x_28, 1); lean_inc(x_29); lean_dec(x_28); x_30 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_30, 0, x_14); -lean_ctor_set(x_30, 1, x_24); -lean_ctor_set(x_30, 2, x_27); +lean_ctor_set(x_30, 0, x_17); +lean_ctor_set(x_30, 1, x_27); +lean_ctor_set(x_30, 2, x_19); lean_ctor_set(x_30, 3, x_29); -lean_ctor_set(x_15, 1, x_8); -lean_ctor_set(x_15, 0, x_30); -return x_15; +lean_ctor_set(x_10, 0, x_30); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_10); +lean_ctor_set(x_31, 1, x_8); +return x_31; +} } else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_31 = lean_ctor_get(x_15, 1); -lean_inc(x_31); -lean_dec(x_15); -x_32 = lean_ctor_get(x_12, 0); +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_32 = lean_ctor_get(x_10, 0); lean_inc(x_32); -lean_dec(x_12); -lean_inc(x_9); -x_33 = l_Lean_FileMap_toPosition(x_9, x_32); +lean_dec(x_10); +x_33 = lean_ctor_get(x_6, 1); +lean_inc(x_33); +lean_dec(x_6); +x_34 = lean_ctor_get(x_32, 0); +lean_inc(x_34); +lean_inc(x_33); +x_35 = l_Lean_FileMap_toPosition(x_33, x_34); +lean_dec(x_34); +x_36 = lean_ctor_get(x_32, 1); +lean_inc(x_36); lean_dec(x_32); lean_inc(x_33); -x_34 = l_Lean_FileMap_leanPosToLspPos(x_9, x_33); -lean_dec(x_9); -x_35 = lean_ctor_get(x_34, 1); +x_37 = l_Lean_FileMap_toPosition(x_33, x_36); +lean_dec(x_36); lean_inc(x_35); -lean_dec(x_34); -x_36 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_36, 0, x_14); -lean_ctor_set(x_36, 1, x_31); -lean_ctor_set(x_36, 2, x_33); -lean_ctor_set(x_36, 3, x_35); -x_37 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_37, 0, x_36); -lean_ctor_set(x_37, 1, x_8); -return x_37; -} -} -} -else -{ -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_11, 0); -lean_inc(x_38); -lean_dec(x_11); -lean_inc(x_9); -x_39 = l_Lean_FileMap_toPosition(x_9, x_38); -lean_dec(x_38); -lean_inc(x_39); -x_40 = l_Lean_FileMap_leanPosToLspPos(x_9, x_39); -if (lean_obj_tag(x_12) == 0) -{ -uint8_t x_41; -lean_dec(x_9); -x_41 = !lean_is_exclusive(x_40); -if (x_41 == 0) -{ -lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_ctor_get(x_40, 1); -x_43 = lean_ctor_get(x_40, 0); -lean_dec(x_43); -lean_inc(x_42); -lean_inc(x_39); -x_44 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_44, 0, x_39); -lean_ctor_set(x_44, 1, x_42); -lean_ctor_set(x_44, 2, x_39); -lean_ctor_set(x_44, 3, x_42); -lean_ctor_set(x_40, 1, x_8); -lean_ctor_set(x_40, 0, x_44); -return x_40; -} -else -{ -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_40, 1); -lean_inc(x_45); -lean_dec(x_40); -lean_inc(x_45); +x_38 = l_Lean_FileMap_leanPosToLspPos(x_33, x_35); +x_39 = lean_ctor_get(x_38, 1); lean_inc(x_39); -x_46 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_46, 0, x_39); -lean_ctor_set(x_46, 1, x_45); -lean_ctor_set(x_46, 2, x_39); -lean_ctor_set(x_46, 3, x_45); -x_47 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_47, 0, x_46); -lean_ctor_set(x_47, 1, x_8); -return x_47; -} -} -else -{ -uint8_t x_48; -x_48 = !lean_is_exclusive(x_40); -if (x_48 == 0) -{ -lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_49 = lean_ctor_get(x_40, 1); -x_50 = lean_ctor_get(x_40, 0); -lean_dec(x_50); -x_51 = lean_ctor_get(x_12, 0); -lean_inc(x_51); -lean_dec(x_12); -lean_inc(x_9); -x_52 = l_Lean_FileMap_toPosition(x_9, x_51); -lean_dec(x_51); -lean_inc(x_52); -x_53 = l_Lean_FileMap_leanPosToLspPos(x_9, x_52); -lean_dec(x_9); -x_54 = lean_ctor_get(x_53, 1); -lean_inc(x_54); -lean_dec(x_53); -x_55 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_55, 0, x_39); -lean_ctor_set(x_55, 1, x_49); -lean_ctor_set(x_55, 2, x_52); -lean_ctor_set(x_55, 3, x_54); -lean_ctor_set(x_40, 1, x_8); -lean_ctor_set(x_40, 0, x_55); -return x_40; +if (lean_is_exclusive(x_38)) { + lean_ctor_release(x_38, 0); + lean_ctor_release(x_38, 1); + x_40 = x_38; +} else { + lean_dec_ref(x_38); + x_40 = lean_box(0); } -else -{ -lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_56 = lean_ctor_get(x_40, 1); -lean_inc(x_56); -lean_dec(x_40); -x_57 = lean_ctor_get(x_12, 0); -lean_inc(x_57); -lean_dec(x_12); -lean_inc(x_9); -x_58 = l_Lean_FileMap_toPosition(x_9, x_57); -lean_dec(x_57); -lean_inc(x_58); -x_59 = l_Lean_FileMap_leanPosToLspPos(x_9, x_58); -lean_dec(x_9); -x_60 = lean_ctor_get(x_59, 1); -lean_inc(x_60); -lean_dec(x_59); -x_61 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_61, 0, x_39); -lean_ctor_set(x_61, 1, x_56); -lean_ctor_set(x_61, 2, x_58); -lean_ctor_set(x_61, 3, x_60); -x_62 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_62, 0, x_61); -lean_ctor_set(x_62, 1, x_8); -return x_62; +lean_inc(x_37); +x_41 = l_Lean_FileMap_leanPosToLspPos(x_33, x_37); +lean_dec(x_33); +x_42 = lean_ctor_get(x_41, 1); +lean_inc(x_42); +lean_dec(x_41); +x_43 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_43, 0, x_35); +lean_ctor_set(x_43, 1, x_39); +lean_ctor_set(x_43, 2, x_37); +lean_ctor_set(x_43, 3, x_42); +x_44 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_44, 0, x_43); +if (lean_is_scalar(x_40)) { + x_45 = lean_alloc_ctor(0, 2, 0); +} else { + x_45 = x_40; } +lean_ctor_set(x_45, 0, x_44); +lean_ctor_set(x_45, 1, x_8); +return x_45; } } } } -static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__1() { +static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__1() { _start: { lean_object* x_1; @@ -43149,7 +43054,7 @@ x_1 = l_Lean_declRangeExt; return x_1; } } -static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__2() { +static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__2() { _start: { lean_object* x_1; @@ -43157,43 +43062,43 @@ x_1 = l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_box(0), lean_box(0)); return x_1; } } -static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__3() { +static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__2; +x_1 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___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_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__4() { +static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__3; +x_1 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__3; x_2 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_2, 0, x_1); lean_ctor_set(x_2, 1, x_1); return x_2; } } -static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__5() { +static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__5() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__3; +x_1 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__3; x_2 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_2, 0, x_1); lean_ctor_set(x_2, 1, x_1); return x_2; } } -static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__6() { +static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__6() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__3; +x_1 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__3; x_2 = lean_alloc_ctor(0, 4, 0); lean_ctor_set(x_2, 0, x_1); lean_ctor_set(x_2, 1, x_1); @@ -43202,13 +43107,13 @@ lean_ctor_set(x_2, 3, x_1); return x_2; } } -static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__7() { +static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__5; -x_2 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__3; -x_3 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__6; +x_1 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__5; +x_2 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__3; +x_3 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__6; x_4 = lean_alloc_ctor(0, 7, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -43220,7 +43125,7 @@ lean_ctor_set(x_4, 6, x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___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_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { lean_object* x_10; uint8_t x_11; @@ -43235,7 +43140,7 @@ x_14 = lean_ctor_get(x_12, 0); lean_inc(x_14); lean_dec(x_12); x_15 = l_Lean_instInhabitedDeclarationRanges; -x_16 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__1; +x_16 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__1; lean_inc(x_1); x_17 = l_Lean_MapDeclarationExtension_contains___rarg(x_15, x_16, x_14, x_1); lean_dec(x_14); @@ -43257,7 +43162,7 @@ x_22 = lean_ctor_get(x_19, 0); x_23 = lean_ctor_get(x_19, 4); lean_dec(x_23); x_24 = l_Lean_MapDeclarationExtension_insert___rarg(x_16, x_22, x_1, x_2); -x_25 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__4; +x_25 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__4; lean_ctor_set(x_19, 4, x_25); lean_ctor_set(x_19, 0, x_24); x_26 = lean_st_ref_set(x_8, x_19, x_20); @@ -43276,7 +43181,7 @@ if (x_31 == 0) lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; x_32 = lean_ctor_get(x_29, 1); lean_dec(x_32); -x_33 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__7; +x_33 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__7; lean_ctor_set(x_29, 1, x_33); x_34 = lean_st_ref_set(x_6, x_29, x_30); x_35 = !lean_is_exclusive(x_34); @@ -43314,7 +43219,7 @@ lean_inc(x_43); lean_inc(x_42); lean_inc(x_41); lean_dec(x_29); -x_45 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__7; +x_45 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__7; x_46 = lean_alloc_ctor(0, 5, 0); lean_ctor_set(x_46, 0, x_41); lean_ctor_set(x_46, 1, x_45); @@ -43360,7 +43265,7 @@ lean_inc(x_53); lean_inc(x_52); lean_dec(x_19); x_58 = l_Lean_MapDeclarationExtension_insert___rarg(x_16, x_52, x_1, x_2); -x_59 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__4; +x_59 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__4; x_60 = lean_alloc_ctor(0, 7, 0); lean_ctor_set(x_60, 0, x_58); lean_ctor_set(x_60, 1, x_53); @@ -43398,7 +43303,7 @@ if (lean_is_exclusive(x_64)) { lean_dec_ref(x_64); x_70 = lean_box(0); } -x_71 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__7; +x_71 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__7; if (lean_is_scalar(x_70)) { x_72 = lean_alloc_ctor(0, 5, 0); } else { @@ -43453,7 +43358,7 @@ x_81 = lean_ctor_get(x_79, 0); lean_inc(x_81); lean_dec(x_79); x_82 = l_Lean_instInhabitedDeclarationRanges; -x_83 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__1; +x_83 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__1; lean_inc(x_1); x_84 = l_Lean_MapDeclarationExtension_contains___rarg(x_82, x_83, x_81, x_1); lean_dec(x_81); @@ -43492,7 +43397,7 @@ if (lean_is_exclusive(x_86)) { x_94 = lean_box(0); } x_95 = l_Lean_MapDeclarationExtension_insert___rarg(x_83, x_88, x_1, x_2); -x_96 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__4; +x_96 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__4; if (lean_is_scalar(x_94)) { x_97 = lean_alloc_ctor(0, 7, 0); } else { @@ -43534,7 +43439,7 @@ if (lean_is_exclusive(x_101)) { lean_dec_ref(x_101); x_107 = lean_box(0); } -x_108 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__7; +x_108 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__7; if (lean_is_scalar(x_107)) { x_109 = lean_alloc_ctor(0, 5, 0); } else { @@ -43580,7 +43485,153 @@ return x_116; } } } -static lean_object* _init_l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__7___closed__1() { +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___at_Lean_Elab_Term_elabMutualDef_go___spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; +lean_inc(x_8); +x_11 = l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Term_elabMutualDef_go___spec__9(x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +if (lean_obj_tag(x_12) == 0) +{ +uint8_t x_13; +lean_dec(x_8); +lean_dec(x_1); +x_13 = !lean_is_exclusive(x_11); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_11, 0); +lean_dec(x_14); +x_15 = lean_box(0); +lean_ctor_set(x_11, 0, x_15); +return x_11; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_11, 1); +lean_inc(x_16); +lean_dec(x_11); +x_17 = lean_box(0); +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set(x_18, 1, x_16); +return x_18; +} +} +else +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_19 = lean_ctor_get(x_11, 1); +lean_inc(x_19); +lean_dec(x_11); +x_20 = lean_ctor_get(x_12, 0); +lean_inc(x_20); +lean_dec(x_12); +lean_inc(x_8); +x_21 = l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Term_elabMutualDef_go___spec__9(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_19); +x_22 = lean_ctor_get(x_21, 0); +lean_inc(x_22); +if (lean_obj_tag(x_22) == 0) +{ +uint8_t x_23; +x_23 = !lean_is_exclusive(x_21); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_21, 1); +x_25 = lean_ctor_get(x_21, 0); +lean_dec(x_25); +lean_inc(x_20); +lean_ctor_set(x_21, 1, x_20); +lean_ctor_set(x_21, 0, x_20); +x_26 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10(x_1, x_21, x_4, x_5, x_6, x_7, x_8, x_9, x_24); +lean_dec(x_8); +return x_26; +} +else +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_21, 1); +lean_inc(x_27); +lean_dec(x_21); +lean_inc(x_20); +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_20); +lean_ctor_set(x_28, 1, x_20); +x_29 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10(x_1, x_28, x_4, x_5, x_6, x_7, x_8, x_9, x_27); +lean_dec(x_8); +return x_29; +} +} +else +{ +uint8_t x_30; +x_30 = !lean_is_exclusive(x_21); +if (x_30 == 0) +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_31 = lean_ctor_get(x_21, 1); +x_32 = lean_ctor_get(x_21, 0); +lean_dec(x_32); +x_33 = lean_ctor_get(x_22, 0); +lean_inc(x_33); +lean_dec(x_22); +lean_ctor_set(x_21, 1, x_33); +lean_ctor_set(x_21, 0, x_20); +x_34 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10(x_1, x_21, x_4, x_5, x_6, x_7, x_8, x_9, x_31); +lean_dec(x_8); +return x_34; +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_35 = lean_ctor_get(x_21, 1); +lean_inc(x_35); +lean_dec(x_21); +x_36 = lean_ctor_get(x_22, 0); +lean_inc(x_36); +lean_dec(x_22); +x_37 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_37, 0, x_20); +lean_ctor_set(x_37, 1, x_36); +x_38 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10(x_1, x_37, x_4, x_5, x_6, x_7, x_8, x_9, x_35); +lean_dec(x_8); +return x_38; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Term_elabMutualDef_go___spec__7___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_12 = lean_box(0); +lean_inc(x_1); +x_13 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_13, 0, x_1); +lean_ctor_set(x_13, 1, x_12); +x_14 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_14, 0, x_2); +lean_ctor_set(x_14, 1, x_13); +x_15 = lean_array_mk(x_14); +x_16 = lean_box(2); +x_17 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders_mkTacTask___closed__10; +x_18 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_18, 0, x_16); +lean_ctor_set(x_18, 1, x_17); +lean_ctor_set(x_18, 2, x_15); +x_19 = l_Lean_Elab_getDeclarationSelectionRef(x_1); +x_20 = l_Lean_Elab_addDeclarationRangesFromSyntax___at_Lean_Elab_Term_elabMutualDef_go___spec__8(x_3, x_18, x_19, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_19); +lean_dec(x_18); +return x_20; +} +} +static lean_object* _init_l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Term_elabMutualDef_go___spec__7___closed__1() { _start: { lean_object* x_1; @@ -43588,84 +43639,50 @@ x_1 = lean_mk_string_unchecked("example", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__7___closed__2() { +static lean_object* _init_l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Term_elabMutualDef_go___spec__7___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders_getBodyTerm_x3f___closed__1; x_2 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders_getBodyTerm_x3f___closed__2; x_3 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders_getBodyTerm_x3f___closed__3; -x_4 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__7___closed__1; +x_4 = l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Term_elabMutualDef_go___spec__7___closed__1; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Term_elabMutualDef_go___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_10; lean_object* x_11; uint8_t x_12; -lean_inc(x_2); -x_10 = l_Lean_Syntax_getKind(x_2); -x_11 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__7___closed__2; -x_12 = lean_name_eq(x_10, x_11); -lean_dec(x_10); -if (x_12 == 0) -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; -lean_inc(x_7); -x_13 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Term_elabMutualDef_go___spec__8(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -x_14 = lean_ctor_get(x_13, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_13, 1); -lean_inc(x_15); -lean_dec(x_13); -x_16 = l_Lean_Elab_getDeclarationSelectionRef(x_2); -lean_inc(x_7); -x_17 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Term_elabMutualDef_go___spec__8(x_16, x_3, x_4, x_5, x_6, x_7, x_8, x_15); -lean_dec(x_16); -x_18 = !lean_is_exclusive(x_17); -if (x_18 == 0) -{ -lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_19 = lean_ctor_get(x_17, 0); -x_20 = lean_ctor_get(x_17, 1); -lean_ctor_set(x_17, 1, x_19); -lean_ctor_set(x_17, 0, x_14); -x_21 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9(x_1, x_17, x_3, x_4, x_5, x_6, x_7, x_8, x_20); -lean_dec(x_7); -return x_21; -} -else +lean_object* x_11; lean_object* x_12; uint8_t x_13; +lean_inc(x_3); +x_11 = l_Lean_Syntax_getKind(x_3); +x_12 = l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Term_elabMutualDef_go___spec__7___closed__2; +x_13 = lean_name_eq(x_11, x_12); +lean_dec(x_11); +if (x_13 == 0) { -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_22 = lean_ctor_get(x_17, 0); -x_23 = lean_ctor_get(x_17, 1); -lean_inc(x_23); -lean_inc(x_22); -lean_dec(x_17); -x_24 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_24, 0, x_14); -lean_ctor_set(x_24, 1, x_22); -x_25 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9(x_1, x_24, x_3, x_4, x_5, x_6, x_7, x_8, x_23); -lean_dec(x_7); -return x_25; -} +lean_object* x_14; lean_object* x_15; +x_14 = lean_box(0); +x_15 = l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Term_elabMutualDef_go___spec__7___lambda__1(x_3, x_2, x_1, x_14, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_15; } else { -lean_object* x_26; lean_object* x_27; -lean_dec(x_7); +lean_object* x_16; lean_object* x_17; +lean_dec(x_8); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_26 = lean_box(0); -x_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_26); -lean_ctor_set(x_27, 1, x_9); -return x_27; +x_16 = lean_box(0); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_16); +lean_ctor_set(x_17, 1, x_10); +return x_17; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__10(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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__11(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; @@ -43709,7 +43726,7 @@ uint8_t x_20; x_20 = !lean_is_exclusive(x_4); if (x_20 == 0) { -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; size_t x_32; size_t x_33; +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; size_t x_34; size_t x_35; x_21 = lean_ctor_get(x_4, 2); lean_dec(x_21); x_22 = lean_ctor_get(x_4, 1); @@ -43727,58 +43744,68 @@ lean_dec(x_24); x_28 = lean_ctor_get(x_27, 1); lean_inc(x_28); lean_dec(x_27); -x_29 = lean_ctor_get(x_14, 0); +x_29 = lean_ctor_get(x_14, 2); lean_inc(x_29); +x_30 = lean_ctor_get(x_29, 0); +lean_inc(x_30); +lean_dec(x_29); +x_31 = lean_ctor_get(x_14, 0); +lean_inc(x_31); lean_dec(x_14); lean_inc(x_9); -x_30 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__7(x_28, x_29, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -x_31 = lean_ctor_get(x_30, 1); -lean_inc(x_31); -lean_dec(x_30); -x_32 = 1; -x_33 = lean_usize_add(x_3, x_32); -x_3 = x_33; -x_11 = x_31; +x_32 = l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Term_elabMutualDef_go___spec__7(x_28, x_30, x_31, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_33 = lean_ctor_get(x_32, 1); +lean_inc(x_33); +lean_dec(x_32); +x_34 = 1; +x_35 = lean_usize_add(x_3, x_34); +x_3 = x_35; +x_11 = x_33; goto _start; } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; size_t x_44; size_t x_45; +lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; size_t x_48; size_t x_49; lean_dec(x_4); -x_35 = lean_array_fget(x_15, x_16); -x_36 = lean_unsigned_to_nat(1u); -x_37 = lean_nat_add(x_16, x_36); +x_37 = lean_array_fget(x_15, x_16); +x_38 = lean_unsigned_to_nat(1u); +x_39 = lean_nat_add(x_16, x_38); lean_dec(x_16); -x_38 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_38, 0, x_15); -lean_ctor_set(x_38, 1, x_37); -lean_ctor_set(x_38, 2, x_17); -x_39 = lean_ctor_get(x_35, 1); -lean_inc(x_39); -lean_dec(x_35); -x_40 = lean_ctor_get(x_39, 1); -lean_inc(x_40); -lean_dec(x_39); -x_41 = lean_ctor_get(x_14, 0); +x_40 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_40, 0, x_15); +lean_ctor_set(x_40, 1, x_39); +lean_ctor_set(x_40, 2, x_17); +x_41 = lean_ctor_get(x_37, 1); lean_inc(x_41); +lean_dec(x_37); +x_42 = lean_ctor_get(x_41, 1); +lean_inc(x_42); +lean_dec(x_41); +x_43 = lean_ctor_get(x_14, 2); +lean_inc(x_43); +x_44 = lean_ctor_get(x_43, 0); +lean_inc(x_44); +lean_dec(x_43); +x_45 = lean_ctor_get(x_14, 0); +lean_inc(x_45); lean_dec(x_14); lean_inc(x_9); -x_42 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__7(x_40, x_41, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -x_43 = lean_ctor_get(x_42, 1); -lean_inc(x_43); -lean_dec(x_42); -x_44 = 1; -x_45 = lean_usize_add(x_3, x_44); -x_3 = x_45; -x_4 = x_38; -x_11 = x_43; +x_46 = l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Term_elabMutualDef_go___spec__7(x_42, x_44, x_45, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_47 = lean_ctor_get(x_46, 1); +lean_inc(x_47); +lean_dec(x_46); +x_48 = 1; +x_49 = lean_usize_add(x_3, x_48); +x_3 = x_49; +x_4 = x_40; +x_11 = x_47; goto _start; } } } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef_go___spec__12(size_t x_1, size_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, 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_Lean_Elab_Term_elabMutualDef_go___spec__13(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; @@ -43812,7 +43839,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__13(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_elabMutualDef_go___spec__14(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; @@ -43847,7 +43874,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__14(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_elabMutualDef_go___spec__15(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; @@ -43882,7 +43909,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Lean_Language_withAlwaysResolvedPromises___at_Lean_Elab_Term_elabMutualDef_go___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_Language_withAlwaysResolvedPromises___at_Lean_Elab_Term_elabMutualDef_go___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_object* x_12; size_t x_13; size_t x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; size_t x_18; lean_object* x_19; @@ -43890,7 +43917,7 @@ x_11 = l_List_iotaTR(x_2); x_12 = lean_array_mk(x_11); x_13 = lean_array_size(x_12); x_14 = 0; -x_15 = l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef_go___spec__12(x_13, x_14, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_15 = l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef_go___spec__13(x_13, x_14, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10); x_16 = lean_ctor_get(x_15, 0); lean_inc(x_16); x_17 = lean_ctor_get(x_15, 1); @@ -43914,7 +43941,7 @@ x_21 = lean_ctor_get(x_19, 1); lean_inc(x_21); lean_dec(x_19); x_22 = lean_box(0); -x_23 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__13(x_1, x_16, x_18, x_14, x_22, x_4, x_5, x_6, x_7, x_8, x_9, x_21); +x_23 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__14(x_1, x_16, x_18, x_14, x_22, x_4, x_5, x_6, x_7, x_8, x_9, x_21); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -43952,7 +43979,7 @@ x_29 = lean_ctor_get(x_19, 1); lean_inc(x_29); lean_dec(x_19); x_30 = lean_box(0); -x_31 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__14(x_1, x_16, x_18, x_14, x_30, x_4, x_5, x_6, x_7, x_8, x_9, x_29); +x_31 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__15(x_1, x_16, x_18, x_14, x_30, 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); @@ -43984,7 +44011,7 @@ return x_35; } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef_go___spec__16(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_Lean_Elab_Term_elabMutualDef_go___spec__17(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; @@ -44018,7 +44045,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__17(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_elabMutualDef_go___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; @@ -44053,7 +44080,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___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) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___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; @@ -44088,7 +44115,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Lean_Language_withAlwaysResolvedPromises___at_Lean_Elab_Term_elabMutualDef_go___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_Language_withAlwaysResolvedPromises___at_Lean_Elab_Term_elabMutualDef_go___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; size_t x_13; size_t x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; size_t x_18; lean_object* x_19; @@ -44096,7 +44123,7 @@ x_11 = l_List_iotaTR(x_2); x_12 = lean_array_mk(x_11); x_13 = lean_array_size(x_12); x_14 = 0; -x_15 = l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef_go___spec__16(x_13, x_14, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_15 = l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef_go___spec__17(x_13, x_14, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10); x_16 = lean_ctor_get(x_15, 0); lean_inc(x_16); x_17 = lean_ctor_get(x_15, 1); @@ -44120,7 +44147,7 @@ x_21 = lean_ctor_get(x_19, 1); lean_inc(x_21); lean_dec(x_19); x_22 = lean_box(0); -x_23 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__17(x_1, x_16, x_18, x_14, x_22, x_4, x_5, x_6, x_7, x_8, x_9, x_21); +x_23 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__18(x_1, x_16, x_18, x_14, x_22, x_4, x_5, x_6, x_7, x_8, x_9, x_21); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -44158,7 +44185,7 @@ x_29 = lean_ctor_get(x_19, 1); lean_inc(x_29); lean_dec(x_19); x_30 = lean_box(0); -x_31 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__18(x_1, x_16, x_18, x_14, x_30, x_4, x_5, x_6, x_7, x_8, x_9, x_29); +x_31 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__19(x_1, x_16, x_18, x_14, x_30, 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); @@ -44516,7 +44543,7 @@ if (x_33 == 0) { lean_object* x_36; uint8_t x_37; lean_dec(x_31); -x_36 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5___closed__1; +x_36 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__7___closed__1; x_37 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_30, x_36); lean_dec(x_30); if (x_37 == 0) @@ -44546,7 +44573,7 @@ x_41 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_elabMutualDef_go___spec__5(x_1 if (x_41 == 0) { lean_object* x_42; uint8_t x_43; -x_42 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5___closed__1; +x_42 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__7___closed__1; x_43 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_30, x_42); lean_dec(x_30); if (x_43 == 0) @@ -45046,7 +45073,7 @@ x_27 = lean_unsigned_to_nat(0u); x_28 = l_Array_toSubarray___rarg(x_20, x_27, x_26); x_29 = lean_array_size(x_1); x_30 = 0; -x_31 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__10(x_1, x_29, x_30, x_28, x_6, x_7, x_8, x_9, x_10, x_11, x_25); +x_31 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__11(x_1, x_29, x_30, x_28, x_6, x_7, x_8, x_9, x_10, x_11, x_25); lean_dec(x_11); lean_dec(x_9); lean_dec(x_8); @@ -45184,7 +45211,7 @@ lean_closure_set(x_13, 1, x_5); lean_closure_set(x_13, 2, x_2); lean_closure_set(x_13, 3, x_3); x_14 = l_Lean_Elab_Tactic_instInhabitedTacticParsedSnapshot; -x_15 = l_Lean_Language_withAlwaysResolvedPromises___at_Lean_Elab_Term_elabMutualDef_go___spec__11(x_14, x_4, x_13, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_15 = l_Lean_Language_withAlwaysResolvedPromises___at_Lean_Elab_Term_elabMutualDef_go___spec__12(x_14, x_4, x_13, x_6, x_7, x_8, x_9, x_10, x_11, x_12); return x_15; } } @@ -45200,7 +45227,7 @@ lean_closure_set(x_13, 0, x_3); lean_closure_set(x_13, 1, x_1); lean_closure_set(x_13, 2, x_2); lean_closure_set(x_13, 3, x_12); -x_14 = l_Lean_Language_withAlwaysResolvedPromises___at_Lean_Elab_Term_elabMutualDef_go___spec__15(x_11, x_12, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_14 = l_Lean_Language_withAlwaysResolvedPromises___at_Lean_Elab_Term_elabMutualDef_go___spec__16(x_11, x_12, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10); return x_14; } } @@ -45293,11 +45320,11 @@ lean_dec(x_4); return x_13; } } -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Term_elabMutualDef_go___spec__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Term_elabMutualDef_go___spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; -x_9 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Term_elabMutualDef_go___spec__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Term_elabMutualDef_go___spec__9(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_7); lean_dec(x_5); lean_dec(x_4); @@ -45307,11 +45334,11 @@ lean_dec(x_1); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___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_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { lean_object* x_10; -x_10 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_10 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__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); @@ -45321,20 +45348,49 @@ lean_dec(x_3); return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___at_Lean_Elab_Term_elabMutualDef_go___spec__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_10; -x_10 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__7(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_8); +lean_object* x_11; +x_11 = l_Lean_Elab_addDeclarationRangesFromSyntax___at_Lean_Elab_Term_elabMutualDef_go___spec__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, 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); -return x_10; +lean_dec(x_2); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Term_elabMutualDef_go___spec__7___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +x_12 = l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Term_elabMutualDef_go___spec__7___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Term_elabMutualDef_go___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Term_elabMutualDef_go___spec__7(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_11; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { size_t x_12; size_t x_13; lean_object* x_14; @@ -45342,7 +45398,7 @@ 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_elabMutualDef_go___spec__10(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_Lean_Elab_Term_elabMutualDef_go___spec__11(x_1, x_12, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_10); lean_dec(x_8); lean_dec(x_7); @@ -45352,7 +45408,7 @@ lean_dec(x_1); return x_14; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef_go___spec__12___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef_go___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: { size_t x_11; size_t x_12; lean_object* x_13; @@ -45360,7 +45416,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_Lean_Elab_Term_elabMutualDef_go___spec__12(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_Lean_Elab_Term_elabMutualDef_go___spec__13(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); @@ -45370,7 +45426,7 @@ lean_dec(x_4); return x_13; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___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_object* x_11, lean_object* x_12) { _start: { size_t x_13; size_t x_14; lean_object* x_15; @@ -45378,7 +45434,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_elabMutualDef_go___spec__13(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_elabMutualDef_go___spec__14(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -45389,7 +45445,7 @@ lean_dec(x_2); return x_15; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___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_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__15___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { size_t x_13; size_t x_14; lean_object* x_15; @@ -45397,7 +45453,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_elabMutualDef_go___spec__14(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_15 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__15(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -45408,7 +45464,7 @@ lean_dec(x_2); return x_15; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef_go___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_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef_go___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) { _start: { size_t x_11; size_t x_12; lean_object* x_13; @@ -45416,7 +45472,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_Lean_Elab_Term_elabMutualDef_go___spec__16(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_Lean_Elab_Term_elabMutualDef_go___spec__17(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); @@ -45426,7 +45482,7 @@ lean_dec(x_4); return x_13; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___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; @@ -45434,7 +45490,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_elabMutualDef_go___spec__17(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_15 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___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_10); lean_dec(x_9); @@ -45445,7 +45501,7 @@ lean_dec(x_2); return x_15; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__18___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___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; @@ -45453,7 +45509,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_elabMutualDef_go___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); +x_15 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___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_10); lean_dec(x_9); @@ -48733,142 +48789,147 @@ return x_24; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, uint8_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -uint8_t x_10; uint8_t x_11; -x_10 = l_Lean_Syntax_isNone(x_1); -x_11 = l_Lean_Syntax_isNone(x_2); -if (x_10 == 0) -{ +uint8_t x_11; uint8_t x_12; +x_11 = l_Lean_Syntax_isNone(x_1); +x_12 = l_Lean_Syntax_isNone(x_2); if (x_11 == 0) { -uint8_t x_12; lean_object* x_13; lean_object* x_14; -x_12 = 1; -x_13 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_13, 0, x_3); -lean_ctor_set(x_13, 1, x_6); -lean_ctor_set_uint8(x_13, sizeof(void*)*2, x_4); -lean_ctor_set_uint8(x_13, sizeof(void*)*2 + 1, x_12); -lean_ctor_set_uint8(x_13, sizeof(void*)*2 + 2, x_5); -lean_ctor_set_uint8(x_13, sizeof(void*)*2 + 3, x_12); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_13); -lean_ctor_set(x_14, 1, x_9); -return x_14; +if (x_12 == 0) +{ +uint8_t x_13; lean_object* x_14; lean_object* x_15; +x_13 = 1; +x_14 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_14, 0, x_3); +lean_ctor_set(x_14, 1, x_4); +lean_ctor_set(x_14, 2, x_7); +lean_ctor_set_uint8(x_14, sizeof(void*)*3, x_5); +lean_ctor_set_uint8(x_14, sizeof(void*)*3 + 1, x_13); +lean_ctor_set_uint8(x_14, sizeof(void*)*3 + 2, x_6); +lean_ctor_set_uint8(x_14, sizeof(void*)*3 + 3, x_13); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_10); +return x_15; } else { -uint8_t x_15; uint8_t x_16; lean_object* x_17; lean_object* x_18; -x_15 = 1; -x_16 = 0; -x_17 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_17, 0, x_3); -lean_ctor_set(x_17, 1, x_6); -lean_ctor_set_uint8(x_17, sizeof(void*)*2, x_4); -lean_ctor_set_uint8(x_17, sizeof(void*)*2 + 1, x_15); -lean_ctor_set_uint8(x_17, sizeof(void*)*2 + 2, x_5); -lean_ctor_set_uint8(x_17, sizeof(void*)*2 + 3, x_16); -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_17); -lean_ctor_set(x_18, 1, x_9); -return x_18; +uint8_t x_16; uint8_t x_17; lean_object* x_18; lean_object* x_19; +x_16 = 1; +x_17 = 0; +x_18 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_18, 0, x_3); +lean_ctor_set(x_18, 1, x_4); +lean_ctor_set(x_18, 2, x_7); +lean_ctor_set_uint8(x_18, sizeof(void*)*3, x_5); +lean_ctor_set_uint8(x_18, sizeof(void*)*3 + 1, x_16); +lean_ctor_set_uint8(x_18, sizeof(void*)*3 + 2, x_6); +lean_ctor_set_uint8(x_18, sizeof(void*)*3 + 3, x_17); +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set(x_19, 1, x_10); +return x_19; } } else { -if (x_11 == 0) +if (x_12 == 0) { -uint8_t x_19; uint8_t x_20; lean_object* x_21; lean_object* x_22; -x_19 = 0; -x_20 = 1; -x_21 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_21, 0, x_3); -lean_ctor_set(x_21, 1, x_6); -lean_ctor_set_uint8(x_21, sizeof(void*)*2, x_4); -lean_ctor_set_uint8(x_21, sizeof(void*)*2 + 1, x_19); -lean_ctor_set_uint8(x_21, sizeof(void*)*2 + 2, x_5); -lean_ctor_set_uint8(x_21, sizeof(void*)*2 + 3, x_20); -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_21); -lean_ctor_set(x_22, 1, x_9); -return x_22; +uint8_t x_20; uint8_t x_21; lean_object* x_22; lean_object* x_23; +x_20 = 0; +x_21 = 1; +x_22 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_22, 0, x_3); +lean_ctor_set(x_22, 1, x_4); +lean_ctor_set(x_22, 2, x_7); +lean_ctor_set_uint8(x_22, sizeof(void*)*3, x_5); +lean_ctor_set_uint8(x_22, sizeof(void*)*3 + 1, x_20); +lean_ctor_set_uint8(x_22, sizeof(void*)*3 + 2, x_6); +lean_ctor_set_uint8(x_22, sizeof(void*)*3 + 3, x_21); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_10); +return x_23; } else { -uint8_t x_23; lean_object* x_24; lean_object* x_25; -x_23 = 0; -x_24 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_24, 0, x_3); -lean_ctor_set(x_24, 1, x_6); -lean_ctor_set_uint8(x_24, sizeof(void*)*2, x_4); -lean_ctor_set_uint8(x_24, sizeof(void*)*2 + 1, x_23); -lean_ctor_set_uint8(x_24, sizeof(void*)*2 + 2, x_5); -lean_ctor_set_uint8(x_24, sizeof(void*)*2 + 3, x_23); -x_25 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_25, 0, x_24); -lean_ctor_set(x_25, 1, x_9); -return x_25; +uint8_t x_24; lean_object* x_25; lean_object* x_26; +x_24 = 0; +x_25 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_25, 0, x_3); +lean_ctor_set(x_25, 1, x_4); +lean_ctor_set(x_25, 2, x_7); +lean_ctor_set_uint8(x_25, sizeof(void*)*3, x_5); +lean_ctor_set_uint8(x_25, sizeof(void*)*3 + 1, x_24); +lean_ctor_set_uint8(x_25, sizeof(void*)*3 + 2, x_6); +lean_ctor_set_uint8(x_25, sizeof(void*)*3 + 3, x_24); +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_10); +return x_26; } } } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, lean_object* x_6, uint8_t x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_10; -x_10 = l_Lean_Syntax_getOptional_x3f(x_5); -if (lean_obj_tag(x_10) == 0) +lean_object* x_11; +x_11 = l_Lean_Syntax_getOptional_x3f(x_6); +if (lean_obj_tag(x_11) == 0) { -lean_object* x_11; lean_object* x_12; -x_11 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___closed__1; -x_12 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__1(x_1, x_2, x_3, x_6, x_4, x_11, x_7, x_8, x_9); -lean_dec(x_7); -return x_12; +lean_object* x_12; lean_object* x_13; +x_12 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___closed__1; +x_13 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_7, x_5, x_12, x_8, x_9, x_10); +lean_dec(x_8); +return x_13; } else { -lean_object* x_13; lean_object* x_14; -x_13 = lean_ctor_get(x_10, 0); -lean_inc(x_13); -lean_dec(x_10); -lean_inc(x_7); -x_14 = l_Lean_Elab_elabDeclAttrs___at_Lean_Elab_Command_elabMutualDef___spec__2(x_13, x_7, x_8, x_9); -lean_dec(x_13); -if (lean_obj_tag(x_14) == 0) +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_11, 0); +lean_inc(x_14); +lean_dec(x_11); +lean_inc(x_8); +x_15 = l_Lean_Elab_elabDeclAttrs___at_Lean_Elab_Command_elabMutualDef___spec__2(x_14, x_8, x_9, x_10); +lean_dec(x_14); +if (lean_obj_tag(x_15) == 0) { -lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = lean_ctor_get(x_14, 0); -lean_inc(x_15); -x_16 = lean_ctor_get(x_14, 1); +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_15, 0); lean_inc(x_16); -lean_dec(x_14); -x_17 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__1(x_1, x_2, x_3, x_6, x_4, x_15, x_7, x_8, x_16); -lean_dec(x_7); -return x_17; +x_17 = lean_ctor_get(x_15, 1); +lean_inc(x_17); +lean_dec(x_15); +x_18 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_7, x_5, x_16, x_8, x_9, x_17); +lean_dec(x_8); +return x_18; } else { -uint8_t x_18; -lean_dec(x_7); +uint8_t x_19; +lean_dec(x_8); +lean_dec(x_4); lean_dec(x_3); -x_18 = !lean_is_exclusive(x_14); -if (x_18 == 0) +x_19 = !lean_is_exclusive(x_15); +if (x_19 == 0) { -return x_14; +return x_15; } else { -lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_19 = lean_ctor_get(x_14, 0); -x_20 = lean_ctor_get(x_14, 1); +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_15, 0); +x_21 = lean_ctor_get(x_15, 1); +lean_inc(x_21); lean_inc(x_20); -lean_inc(x_19); -lean_dec(x_14); -x_21 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_21, 0, x_19); -lean_ctor_set(x_21, 1, x_20); -return x_21; +lean_dec(x_15); +x_22 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_22, 0, x_20); +lean_ctor_set(x_22, 1, x_21); +return x_22; } } } @@ -48931,77 +48992,78 @@ x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_10; -x_10 = l_Lean_Syntax_getOptional_x3f(x_5); -if (lean_obj_tag(x_10) == 0) +lean_object* x_11; +x_11 = l_Lean_Syntax_getOptional_x3f(x_6); +if (lean_obj_tag(x_11) == 0) { -uint8_t x_11; lean_object* x_12; -x_11 = 0; -x_12 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__2(x_1, x_2, x_6, x_3, x_4, x_11, x_7, x_8, x_9); -return x_12; +uint8_t x_12; lean_object* x_13; +x_12 = 0; +x_13 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__2(x_1, x_2, x_3, x_7, x_4, x_5, x_12, x_8, x_9, x_10); +return x_13; } else { -lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; -x_13 = lean_ctor_get(x_10, 0); -lean_inc(x_13); -lean_dec(x_10); -lean_inc(x_13); -x_14 = l_Lean_Syntax_getKind(x_13); -x_15 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3___closed__2; -x_16 = lean_name_eq(x_14, x_15); -if (x_16 == 0) +lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_14 = lean_ctor_get(x_11, 0); +lean_inc(x_14); +lean_dec(x_11); +lean_inc(x_14); +x_15 = l_Lean_Syntax_getKind(x_14); +x_16 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3___closed__2; +x_17 = lean_name_eq(x_15, x_16); +if (x_17 == 0) { -lean_object* x_17; uint8_t x_18; -x_17 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3___closed__4; -x_18 = lean_name_eq(x_14, x_17); -lean_dec(x_14); -if (x_18 == 0) +lean_object* x_18; uint8_t x_19; +x_18 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3___closed__4; +x_19 = lean_name_eq(x_15, x_18); +lean_dec(x_15); +if (x_19 == 0) { -lean_object* x_19; lean_object* x_20; uint8_t x_21; -lean_dec(x_6); -x_19 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3___closed__6; -x_20 = l_Lean_throwErrorAt___at_Lean_Elab_Command_elabMutualDef___spec__7(x_13, x_19, x_7, x_8, x_9); -lean_dec(x_13); -x_21 = !lean_is_exclusive(x_20); -if (x_21 == 0) +lean_object* x_20; lean_object* x_21; uint8_t x_22; +lean_dec(x_7); +lean_dec(x_3); +x_20 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3___closed__6; +x_21 = l_Lean_throwErrorAt___at_Lean_Elab_Command_elabMutualDef___spec__7(x_14, x_20, x_8, x_9, x_10); +lean_dec(x_14); +x_22 = !lean_is_exclusive(x_21); +if (x_22 == 0) { -return x_20; +return x_21; } else { -lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_22 = lean_ctor_get(x_20, 0); -x_23 = lean_ctor_get(x_20, 1); +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_21, 0); +x_24 = lean_ctor_get(x_21, 1); +lean_inc(x_24); lean_inc(x_23); -lean_inc(x_22); -lean_dec(x_20); -x_24 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_24, 0, x_22); -lean_ctor_set(x_24, 1, x_23); -return x_24; +lean_dec(x_21); +x_25 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +return x_25; } } else { -uint8_t x_25; lean_object* x_26; -lean_dec(x_13); -x_25 = 1; -x_26 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__2(x_1, x_2, x_6, x_3, x_4, x_25, x_7, x_8, x_9); -return x_26; +uint8_t x_26; lean_object* x_27; +lean_dec(x_14); +x_26 = 1; +x_27 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__2(x_1, x_2, x_3, x_7, x_4, x_5, x_26, x_8, x_9, x_10); +return x_27; } } else { -uint8_t x_27; lean_object* x_28; +uint8_t x_28; lean_object* x_29; +lean_dec(x_15); lean_dec(x_14); -lean_dec(x_13); -x_27 = 2; -x_28 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__2(x_1, x_2, x_6, x_3, x_4, x_27, x_7, x_8, x_9); -return x_28; +x_28 = 2; +x_29 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__2(x_1, x_2, x_3, x_7, x_4, x_5, x_28, x_8, x_9, x_10); +return x_29; } } } @@ -49083,7 +49145,7 @@ if (lean_obj_tag(x_18) == 0) { lean_object* x_20; lean_object* x_21; x_20 = lean_box(0); -x_21 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3(x_12, x_14, x_19, x_8, x_10, x_20, x_2, x_3, x_4); +x_21 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3(x_12, x_14, x_1, x_19, x_8, x_10, x_20, x_2, x_3, x_4); lean_dec(x_10); lean_dec(x_8); lean_dec(x_14); @@ -49110,7 +49172,7 @@ x_26 = lean_ctor_get(x_24, 1); lean_inc(x_26); lean_dec(x_24); lean_ctor_set(x_18, 0, x_25); -x_27 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3(x_12, x_14, x_19, x_8, x_10, x_18, x_2, x_3, x_26); +x_27 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3(x_12, x_14, x_1, x_19, x_8, x_10, x_18, x_2, x_3, x_26); lean_dec(x_10); lean_dec(x_8); lean_dec(x_14); @@ -49126,6 +49188,7 @@ lean_dec(x_12); lean_dec(x_10); lean_dec(x_8); lean_dec(x_2); +lean_dec(x_1); x_28 = !lean_is_exclusive(x_24); if (x_28 == 0) { @@ -49165,7 +49228,7 @@ lean_inc(x_35); lean_dec(x_33); x_36 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_36, 0, x_34); -x_37 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3(x_12, x_14, x_19, x_8, x_10, x_36, x_2, x_3, x_35); +x_37 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3(x_12, x_14, x_1, x_19, x_8, x_10, x_36, x_2, x_3, x_35); lean_dec(x_10); lean_dec(x_8); lean_dec(x_14); @@ -49180,6 +49243,7 @@ lean_dec(x_12); lean_dec(x_10); lean_dec(x_8); lean_dec(x_2); +lean_dec(x_1); x_38 = lean_ctor_get(x_33, 0); lean_inc(x_38); x_39 = lean_ctor_get(x_33, 1); @@ -49750,6 +49814,7 @@ lean_ctor_set(x_25, 1, x_43); x_44 = lean_array_fget(x_1, x_10); x_45 = l_Lean_Syntax_getArg(x_44, x_18); lean_inc(x_13); +lean_inc(x_45); x_46 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1(x_45, x_13, x_14, x_15); if (lean_obj_tag(x_46) == 0) { @@ -50047,6 +50112,7 @@ lean_ctor_set(x_99, 2, x_35); x_100 = lean_array_fget(x_1, x_10); x_101 = l_Lean_Syntax_getArg(x_100, x_18); lean_inc(x_13); +lean_inc(x_101); x_102 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1(x_101, x_13, x_14, x_15); if (lean_obj_tag(x_102) == 0) { @@ -50393,6 +50459,7 @@ lean_ctor_set(x_160, 2, x_153); x_161 = lean_array_fget(x_1, x_10); x_162 = l_Lean_Syntax_getArg(x_161, x_18); lean_inc(x_13); +lean_inc(x_162); x_163 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1(x_162, x_13, x_14, x_15); if (lean_obj_tag(x_163) == 0) { @@ -50756,6 +50823,7 @@ lean_ctor_set(x_224, 2, x_216); x_225 = lean_array_fget(x_1, x_10); x_226 = l_Lean_Syntax_getArg(x_225, x_18); lean_inc(x_13); +lean_inc(x_226); x_227 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1(x_226, x_13, x_14, x_15); if (lean_obj_tag(x_227) == 0) { @@ -51135,6 +51203,7 @@ lean_ctor_set(x_291, 2, x_282); x_292 = lean_array_fget(x_1, x_10); x_293 = l_Lean_Syntax_getArg(x_292, x_18); lean_inc(x_13); +lean_inc(x_293); x_294 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1(x_293, x_13, x_14, x_15); if (lean_obj_tag(x_294) == 0) { @@ -51434,48 +51503,55 @@ return x_341; } } } -LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Elab_Command_elabMutualDef___spec__10(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Elab_Command_elabMutualDef___spec__10___lambda__1(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_3; uint8_t x_4; -lean_inc(x_2); -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -x_4 = !lean_is_exclusive(x_2); -if (x_4 == 0) +uint8_t x_3; +x_3 = !lean_is_exclusive(x_1); +if (x_3 == 0) { -lean_object* x_5; size_t x_6; size_t x_7; lean_object* x_8; lean_object* x_9; -x_5 = lean_ctor_get(x_2, 1); -x_6 = lean_array_size(x_5); -x_7 = 0; -x_8 = l_Array_mapMUnsafe_map___at_Lean_Elab_instToSnapshotTreeDefsParsedSnapshot___spec__1(x_6, x_7, x_5); -lean_ctor_set(x_2, 1, x_8); -x_9 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_9, 0, x_3); -lean_ctor_set(x_9, 1, x_2); -return x_9; +lean_object* x_4; size_t x_5; size_t x_6; lean_object* x_7; +x_4 = lean_ctor_get(x_1, 1); +x_5 = lean_array_size(x_4); +x_6 = 0; +x_7 = l_Array_mapMUnsafe_map___at_Lean_Elab_instToSnapshotTreeDefsParsedSnapshot___spec__1(x_5, x_6, x_4); +lean_ctor_set(x_1, 1, x_7); +return x_1; } else { -lean_object* x_10; lean_object* x_11; size_t x_12; size_t x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_10 = lean_ctor_get(x_2, 0); -x_11 = lean_ctor_get(x_2, 1); -lean_inc(x_11); -lean_inc(x_10); -lean_dec(x_2); -x_12 = lean_array_size(x_11); -x_13 = 0; -x_14 = l_Array_mapMUnsafe_map___at_Lean_Elab_instToSnapshotTreeDefsParsedSnapshot___spec__1(x_12, x_13, x_11); -x_15 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_15, 0, x_10); -lean_ctor_set(x_15, 1, x_14); -x_16 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_16, 0, x_3); -lean_ctor_set(x_16, 1, x_15); -return x_16; +lean_object* x_8; lean_object* x_9; size_t x_10; size_t x_11; lean_object* x_12; lean_object* x_13; +x_8 = lean_ctor_get(x_1, 0); +x_9 = lean_ctor_get(x_1, 1); +lean_inc(x_9); +lean_inc(x_8); +lean_dec(x_1); +x_10 = lean_array_size(x_9); +x_11 = 0; +x_12 = l_Array_mapMUnsafe_map___at_Lean_Elab_instToSnapshotTreeDefsParsedSnapshot___spec__1(x_10, x_11, x_9); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_8); +lean_ctor_set(x_13, 1, x_12); +return x_13; +} } } +LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Elab_Command_elabMutualDef___spec__10(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +lean_inc(x_2); +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +x_4 = lean_alloc_closure((void*)(l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Elab_Command_elabMutualDef___spec__10___lambda__1___boxed), 2, 1); +lean_closure_set(x_4, 0, x_2); +x_5 = lean_mk_thunk(x_4); +x_6 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_6, 0, x_3); +lean_ctor_set(x_6, 1, x_5); +return x_6; +} } LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabMutualDef___spec__12(size_t x_1, size_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: @@ -52044,51 +52120,51 @@ lean_dec(x_1); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -uint8_t x_10; uint8_t x_11; lean_object* x_12; -x_10 = lean_unbox(x_4); -lean_dec(x_4); +uint8_t x_11; uint8_t x_12; lean_object* x_13; x_11 = lean_unbox(x_5); lean_dec(x_5); -x_12 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__1(x_1, x_2, x_3, x_10, x_11, x_6, x_7, x_8, x_9); +x_12 = lean_unbox(x_6); +lean_dec(x_6); +x_13 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_11, x_12, x_7, x_8, x_9, x_10); +lean_dec(x_9); lean_dec(x_8); -lean_dec(x_7); lean_dec(x_2); lean_dec(x_1); -return x_12; +return x_13; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -uint8_t x_10; uint8_t x_11; lean_object* x_12; -x_10 = lean_unbox(x_4); -lean_dec(x_4); -x_11 = lean_unbox(x_6); -lean_dec(x_6); -x_12 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__2(x_1, x_2, x_3, x_10, x_5, x_11, x_7, x_8, x_9); -lean_dec(x_8); +uint8_t x_11; uint8_t x_12; lean_object* x_13; +x_11 = lean_unbox(x_5); lean_dec(x_5); +x_12 = lean_unbox(x_7); +lean_dec(x_7); +x_13 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__2(x_1, x_2, x_3, x_4, x_11, x_6, x_12, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_6); lean_dec(x_2); lean_dec(x_1); -return x_12; +return x_13; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -uint8_t x_10; lean_object* x_11; -x_10 = lean_unbox(x_3); -lean_dec(x_3); -x_11 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3(x_1, x_2, x_10, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_8); -lean_dec(x_5); +uint8_t x_11; lean_object* x_12; +x_11 = lean_unbox(x_4); lean_dec(x_4); +x_12 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3(x_1, x_2, x_3, x_11, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_5); lean_dec(x_2); lean_dec(x_1); -return x_11; +return x_12; } } LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { @@ -52097,7 +52173,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMu lean_object* x_5; x_5 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1(x_1, x_2, x_3, x_4); lean_dec(x_3); -lean_dec(x_1); return x_5; } } @@ -52143,6 +52218,15 @@ lean_dec(x_1); return x_16; } } +LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Elab_Command_elabMutualDef___spec__10___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Elab_Command_elabMutualDef___spec__10___lambda__1(x_1, x_2); +lean_dec(x_2); +return x_3; +} +} LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabMutualDef___spec__12___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { @@ -52208,7 +52292,7 @@ lean_dec(x_2); return x_9; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__1() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -52218,27 +52302,27 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__2() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__1; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__1; x_2 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__6___lambda__5___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__3() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__2; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__2; x_2 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders_getBodyTerm_x3f___closed__3; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__4() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__4() { _start: { lean_object* x_1; @@ -52246,17 +52330,17 @@ x_1 = lean_mk_string_unchecked("initFn", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__5() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__3; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__4; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__3; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__4; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__6() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__6() { _start: { lean_object* x_1; @@ -52264,47 +52348,47 @@ x_1 = lean_mk_string_unchecked("_@", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__7() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__5; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__6; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__5; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__8() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__7; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__7; x_2 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders_getBodyTerm_x3f___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__9() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__8; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__8; x_2 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__6___lambda__5___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__10() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__9; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__9; x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__12___lambda__2___closed__5; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__11() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__11() { _start: { lean_object* x_1; @@ -52312,33 +52396,33 @@ x_1 = lean_mk_string_unchecked("_hyg", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__12() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__10; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__11; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__10; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__11; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__13() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__12; -x_2 = lean_unsigned_to_nat(16476u); +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__12; +x_2 = lean_unsigned_to_nat(16497u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497_(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; x_2 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkClosureForAux___closed__2; x_3 = 0; -x_4 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__13; +x_4 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__13; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); return x_5; } @@ -52821,34 +52905,38 @@ l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Ela lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__1); l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__2 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__2(); lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__2); -l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__3 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__3(); -lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__3); -l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__4 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__4(); -lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__4); -l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__5 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__5(); -lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__5); -l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__6 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__6(); -lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__6); -l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__7 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__7(); -lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__7); -l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__8 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__8(); -lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__8); -l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__9 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__9(); -lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__9); -l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__10 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__10(); -lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__10); -l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__11 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__11(); -lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__11); -l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__12 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__12(); -lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__12); -l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__13 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__13(); -lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__13); -l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__14 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__14(); -lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__14); -l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__15 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__15(); -lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__15); -l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5___closed__1 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5___closed__1(); -lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5___closed__1); +l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__1 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__1(); +lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__1); +l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__2 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__2(); +lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__2); +l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__3 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__3(); +lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__3); +l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__4 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__4(); +lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__4); +l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__5 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__5(); +lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__5); +l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__6 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__6(); +lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__6); +l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__7 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__7(); +lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__7); +l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__8 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__8(); +lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__8); +l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__9 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__9(); +lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__9); +l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__10 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__10(); +lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__10); +l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__11 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__11(); +lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__11); +l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__12 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__12(); +lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__12); +l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__13 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__13(); +lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__13); +l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__14 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__14(); +lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__14); +l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__15 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__15(); +lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__15); +l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__7___closed__1 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__7___closed__1(); +lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__7___closed__1); l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__18___lambda__1___closed__1 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__18___lambda__1___closed__1(); lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__18___lambda__1___closed__1); l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__18___lambda__1___closed__2 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__18___lambda__1___closed__2(); @@ -52928,24 +53016,24 @@ l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__4___closed lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__4___closed__1); l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__4___closed__2 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__4___closed__2(); lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__4___closed__2); -l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__1 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__1(); -lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__1); -l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__2 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__2(); -lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__2); -l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__3 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__3(); -lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__3); -l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__4 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__4(); -lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__4); -l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__5 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__5(); -lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__5); -l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__6 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__6(); -lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__6); -l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__7 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__7(); -lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__7); -l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__7___closed__1 = _init_l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__7___closed__1(); -lean_mark_persistent(l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__7___closed__1); -l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__7___closed__2 = _init_l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__7___closed__2(); -lean_mark_persistent(l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__7___closed__2); +l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__1 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__1(); +lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__1); +l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__2 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__2(); +lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__2); +l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__3 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__3(); +lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__3); +l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__4 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__4(); +lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__4); +l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__5 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__5(); +lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__5); +l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__6 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__6(); +lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__6); +l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__7 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__7(); +lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__10___closed__7); +l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Term_elabMutualDef_go___spec__7___closed__1 = _init_l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Term_elabMutualDef_go___spec__7___closed__1(); +lean_mark_persistent(l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Term_elabMutualDef_go___spec__7___closed__1); +l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Term_elabMutualDef_go___spec__7___closed__2 = _init_l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Term_elabMutualDef_go___spec__7___closed__2(); +lean_mark_persistent(l_Lean_Elab_addDeclarationRangesForBuiltin___at_Lean_Elab_Term_elabMutualDef_go___spec__7___closed__2); l_Lean_Elab_withSaveInfoContext___at_Lean_Elab_Term_elabMutualDef___spec__1___closed__1 = _init_l_Lean_Elab_withSaveInfoContext___at_Lean_Elab_Term_elabMutualDef___spec__1___closed__1(); lean_mark_persistent(l_Lean_Elab_withSaveInfoContext___at_Lean_Elab_Term_elabMutualDef___spec__1___closed__1); l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualDef___spec__4___lambda__2___closed__1 = _init_l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualDef___spec__4___lambda__2___closed__1(); @@ -52994,33 +53082,33 @@ l_Lean_Elab_Command_elabMutualDef___lambda__3___closed__4 = _init_l_Lean_Elab_Co lean_mark_persistent(l_Lean_Elab_Command_elabMutualDef___lambda__3___closed__4); l_Lean_Elab_Command_elabMutualDef___lambda__3___closed__5 = _init_l_Lean_Elab_Command_elabMutualDef___lambda__3___closed__5(); lean_mark_persistent(l_Lean_Elab_Command_elabMutualDef___lambda__3___closed__5); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__1 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__1(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__1); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__2 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__2(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__2); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__3 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__3(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__3); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__4 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__4(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__4); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__5 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__5(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__5); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__6 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__6(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__6); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__7 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__7(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__7); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__8 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__8(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__8); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__9 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__9(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__9); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__10 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__10(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__10); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__11 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__11(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__11); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__12 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__12(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__12); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__13 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__13(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__13); -if (builtin) {res = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476_(lean_io_mk_world()); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__1 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__1(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__1); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__2 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__2(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__2); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__3 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__3(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__3); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__4 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__4(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__4); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__5 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__5(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__5); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__6 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__6(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__6); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__7 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__7(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__7); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__8 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__8(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__8); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__9 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__9(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__9); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__10 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__10(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__10); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__11 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__11(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__11); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__12 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__12(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__12); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__13 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__13(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497____closed__13); +if (builtin) {res = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16497_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }return lean_io_result_mk_ok(lean_box(0)); diff --git a/stage0/stdlib/Lean/Elab/ParseImportsFast.c b/stage0/stdlib/Lean/Elab/ParseImportsFast.c index c8420f76784d..fc818edba4d9 100644 --- a/stage0/stdlib/Lean/Elab/ParseImportsFast.c +++ b/stage0/stdlib/Lean/Elab/ParseImportsFast.c @@ -14,6 +14,7 @@ extern "C" { #endif lean_object* lean_string_utf8_extract(lean_object*, lean_object*, lean_object*); +lean_object* l_Array_take___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParseImports_isIdCont___boxed(lean_object*, lean_object*); lean_object* l_Lean_Json_compress(lean_object*); uint32_t lean_string_utf8_get(lean_object*, lean_object*); @@ -35,6 +36,7 @@ static lean_object* l_Lean_ParseImports_instInhabitedState___closed__1; LEAN_EXPORT lean_object* l_Lean_ParseImports_moduleIdent_parse(uint8_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParseImports_isIdRestFast___boxed(lean_object*); extern uint32_t l_Lean_idBeginEscape; +lean_object* l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParseImports_keywordCore_go___at_Lean_ParseImports_main___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParseImports_many___at_Lean_ParseImports_main___spec__3___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParseImports_keywordCore_go___at_Lean_ParseImports_preludeOpt___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -83,7 +85,6 @@ LEAN_EXPORT lean_object* l_Lean_ParseImports_many(lean_object*, lean_object*, le LEAN_EXPORT lean_object* l_Lean_ParseImports_keyword(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_ParseImports_State_mkEOIError___closed__2; LEAN_EXPORT lean_object* l_Lean_ParseImports_State_mkEOIError(lean_object*); -lean_object* l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); lean_object* l_IO_FS_readFile(lean_object*, lean_object*); uint8_t l_Lean_isLetterLike(uint32_t); LEAN_EXPORT lean_object* l_Lean_ParseImports_moduleIdent_parse___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -110,7 +111,6 @@ LEAN_EXPORT lean_object* l_Lean_ParseImports_finishCommentBlock_eoi(lean_object* LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_printImportsJson___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_uint32_dec_eq(uint32_t, uint32_t); LEAN_EXPORT lean_object* l_Lean_ParseImports_keywordCore_go___at_Lean_ParseImports_preludeOpt___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Array_shrink___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParseImports_main___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_parseImports_x27(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_ParseImportsFast_0__Lean_toJsonPrintImportResult____x40_Lean_Elab_ParseImportsFast___hyg_1474____closed__1; @@ -3549,7 +3549,7 @@ lean_dec(x_1); x_14 = lean_ctor_get(x_7, 0); lean_inc(x_14); lean_dec(x_7); -x_15 = l_Array_shrink___rarg(x_14, x_6); +x_15 = l_Array_take___rarg(x_14, x_6); lean_dec(x_6); x_16 = lean_box(0); lean_ctor_set(x_3, 2, x_16); @@ -3579,7 +3579,7 @@ lean_dec(x_1); x_19 = lean_ctor_get(x_7, 0); lean_inc(x_19); lean_dec(x_7); -x_20 = l_Array_shrink___rarg(x_19, x_6); +x_20 = l_Array_take___rarg(x_19, x_6); lean_dec(x_6); x_21 = lean_box(0); x_22 = lean_alloc_ctor(0, 3, 0); @@ -4027,7 +4027,7 @@ lean_dec(x_1); x_19 = lean_ctor_get(x_16, 0); lean_inc(x_19); lean_dec(x_16); -x_20 = l_Array_shrink___rarg(x_19, x_6); +x_20 = l_Array_take___rarg(x_19, x_6); lean_dec(x_6); x_21 = lean_box(0); lean_ctor_set(x_3, 2, x_21); @@ -4043,7 +4043,7 @@ lean_dec(x_1); x_22 = lean_ctor_get(x_8, 0); lean_inc(x_22); lean_dec(x_8); -x_23 = l_Array_shrink___rarg(x_22, x_6); +x_23 = l_Array_take___rarg(x_22, x_6); lean_dec(x_6); x_24 = lean_box(0); lean_ctor_set(x_3, 2, x_24); @@ -4082,7 +4082,7 @@ lean_dec(x_1); x_31 = lean_ctor_get(x_28, 0); lean_inc(x_31); lean_dec(x_28); -x_32 = l_Array_shrink___rarg(x_31, x_6); +x_32 = l_Array_take___rarg(x_31, x_6); lean_dec(x_6); x_33 = lean_box(0); x_34 = lean_alloc_ctor(0, 3, 0); @@ -4100,7 +4100,7 @@ lean_dec(x_1); x_35 = lean_ctor_get(x_8, 0); lean_inc(x_35); lean_dec(x_8); -x_36 = l_Array_shrink___rarg(x_35, x_6); +x_36 = l_Array_take___rarg(x_35, x_6); lean_dec(x_6); x_37 = lean_box(0); x_38 = lean_alloc_ctor(0, 3, 0); @@ -4366,7 +4366,7 @@ x_17 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_17, 0, x_10); lean_ctor_set(x_17, 1, x_16); x_18 = l_Lean_parseImports_x27___closed__1; -x_19 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_17, x_18); +x_19 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_17, x_18); x_20 = l_Lean_Json_mkObj(x_19); return x_20; } @@ -4550,7 +4550,7 @@ x_15 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_15, 0, x_4); lean_ctor_set(x_15, 1, x_14); x_16 = l_Lean_parseImports_x27___closed__1; -x_17 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_15, x_16); +x_17 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_15, x_16); x_18 = l_Lean_Json_mkObj(x_17); return x_18; } @@ -4641,7 +4641,7 @@ x_10 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_10, 0, x_9); lean_ctor_set(x_10, 1, x_8); x_11 = l_Lean_parseImports_x27___closed__1; -x_12 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_10, x_11); +x_12 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_10, x_11); x_13 = l_Lean_Json_mkObj(x_12); return x_13; } diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/Basic.c b/stage0/stdlib/Lean/Elab/PreDefinition/Basic.c index 8ec45e86bfc0..a440720bc310 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/Basic.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/Basic.c @@ -55,7 +55,6 @@ extern lean_object* l_Lean_noncomputableExt; lean_object* lean_array_push(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_Basic_0__Lean_Elab_compileDecl___closed__1; LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_fixLevelParams___spec__3___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -uint8_t l_Array_contains___at_Lean_findField_x3f___spec__1(lean_object*, lean_object*); lean_object* l___private_Lean_Util_Trace_0__Lean_addTraceNode___at_Lean_Elab_Term_mkCoe___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_mk_array(lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); @@ -285,6 +284,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_shareCommonPreDefs___lambda__2___boxed(lean LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Basic_0__Lean_Elab_addNonRecAux(lean_object*, uint8_t, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_withTraceNode___at_Lean_Elab_fixLevelParams___spec__3___lambda__4___closed__3; LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_Elab_fixLevelParams___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_instantiateMVarsAtPreDecls___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_Expr_numApps(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Basic_0__Lean_Elab_compileDecl___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -324,7 +324,6 @@ LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_checkCodomainsLev LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_fixLevelParams___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_addAndCompilePartialRec___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_ensureNoRecFn(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_addAndCompilePartialRec___spec__2___closed__1; lean_object* lean_array_uget(lean_object*, size_t); size_t lean_array_size(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Basic_0__Lean_Elab_compileDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -403,20 +402,22 @@ return x_2; static lean_object* _init_l_Lean_Elab_instInhabitedPreDefinition___closed__2() { _start: { -lean_object* x_1; uint8_t x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; +lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; uint8_t x_5; lean_object* x_6; lean_object* x_7; x_1 = lean_box(0); -x_2 = 0; +x_2 = lean_box(0); x_3 = 0; x_4 = 0; -x_5 = l_Lean_Elab_instInhabitedPreDefinition___closed__1; -x_6 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_6, 0, x_1); -lean_ctor_set(x_6, 1, x_5); -lean_ctor_set_uint8(x_6, sizeof(void*)*2, x_2); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 1, x_3); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 2, x_4); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 3, x_3); -return x_6; +x_5 = 0; +x_6 = l_Lean_Elab_instInhabitedPreDefinition___closed__1; +x_7 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_7, 0, x_2); +lean_ctor_set(x_7, 1, x_1); +lean_ctor_set(x_7, 2, x_6); +lean_ctor_set_uint8(x_7, sizeof(void*)*3, x_3); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 1, x_4); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 2, x_5); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 3, x_4); +return x_7; } } static lean_object* _init_l_Lean_Elab_instInhabitedPreDefinition___closed__3() { @@ -2919,7 +2920,7 @@ lean_inc(x_16); x_17 = lean_ctor_get(x_15, 2); lean_inc(x_17); lean_dec(x_15); -x_18 = lean_ctor_get(x_17, 1); +x_18 = lean_ctor_get(x_17, 2); lean_inc(x_18); lean_dec(x_17); lean_inc(x_11); @@ -3468,7 +3469,7 @@ lean_ctor_set(x_11, 0, x_8); lean_ctor_set(x_11, 1, x_9); lean_ctor_set(x_11, 2, x_10); x_12 = lean_ctor_get(x_1, 2); -x_13 = lean_ctor_get_uint8(x_12, sizeof(void*)*2 + 3); +x_13 = lean_ctor_get_uint8(x_12, sizeof(void*)*3 + 3); x_14 = lean_alloc_ctor(0, 1, 1); lean_ctor_set(x_14, 0, x_11); lean_ctor_set_uint8(x_14, sizeof(void*)*1, x_13); @@ -3558,7 +3559,7 @@ if (x_3 == 0) { lean_object* x_4; uint8_t x_5; x_4 = lean_ctor_get(x_1, 2); -x_5 = lean_ctor_get_uint8(x_4, sizeof(void*)*2 + 1); +x_5 = lean_ctor_get_uint8(x_4, sizeof(void*)*3 + 1); if (x_5 == 0) { uint8_t x_6; @@ -7133,7 +7134,7 @@ if (lean_obj_tag(x_23) == 0) lean_object* x_24; uint8_t x_25; x_24 = lean_ctor_get(x_1, 2); lean_inc(x_24); -x_25 = lean_ctor_get_uint8(x_24, sizeof(void*)*2 + 1); +x_25 = lean_ctor_get_uint8(x_24, sizeof(void*)*3 + 1); lean_dec(x_24); if (x_25 == 0) { @@ -7523,7 +7524,7 @@ x_40 = lean_ctor_get(x_17, 5); lean_inc(x_40); x_41 = lean_ctor_get(x_17, 2); lean_inc(x_41); -x_42 = lean_ctor_get_uint8(x_41, sizeof(void*)*2 + 3); +x_42 = lean_ctor_get_uint8(x_41, sizeof(void*)*3 + 3); lean_dec(x_41); x_43 = lean_alloc_ctor(0, 3, 1); lean_ctor_set(x_43, 0, x_39); @@ -7553,7 +7554,7 @@ lean_ctor_set(x_50, 1, x_48); lean_ctor_set(x_50, 2, x_49); x_51 = lean_ctor_get(x_17, 2); lean_inc(x_51); -x_52 = lean_ctor_get_uint8(x_51, sizeof(void*)*2 + 3); +x_52 = lean_ctor_get_uint8(x_51, sizeof(void*)*3 + 3); lean_dec(x_51); if (x_52 == 0) { @@ -7630,7 +7631,7 @@ x_79 = lean_alloc_ctor(2, 0, 4); lean_ctor_set_uint32(x_79, 0, x_78); x_80 = lean_ctor_get(x_17, 2); lean_inc(x_80); -x_81 = lean_ctor_get_uint8(x_80, sizeof(void*)*2 + 3); +x_81 = lean_ctor_get_uint8(x_80, sizeof(void*)*3 + 3); lean_dec(x_80); if (x_81 == 0) { @@ -7846,7 +7847,7 @@ x_134 = lean_ctor_get(x_111, 5); lean_inc(x_134); x_135 = lean_ctor_get(x_111, 2); lean_inc(x_135); -x_136 = lean_ctor_get_uint8(x_135, sizeof(void*)*2 + 3); +x_136 = lean_ctor_get_uint8(x_135, sizeof(void*)*3 + 3); lean_dec(x_135); x_137 = lean_alloc_ctor(0, 3, 1); lean_ctor_set(x_137, 0, x_133); @@ -7876,7 +7877,7 @@ lean_ctor_set(x_144, 1, x_142); lean_ctor_set(x_144, 2, x_143); x_145 = lean_ctor_get(x_111, 2); lean_inc(x_145); -x_146 = lean_ctor_get_uint8(x_145, sizeof(void*)*2 + 3); +x_146 = lean_ctor_get_uint8(x_145, sizeof(void*)*3 + 3); lean_dec(x_145); if (x_146 == 0) { @@ -7953,7 +7954,7 @@ x_173 = lean_alloc_ctor(2, 0, 4); lean_ctor_set_uint32(x_173, 0, x_172); x_174 = lean_ctor_get(x_111, 2); lean_inc(x_174); -x_175 = lean_ctor_get_uint8(x_174, sizeof(void*)*2 + 3); +x_175 = lean_ctor_get_uint8(x_174, sizeof(void*)*3 + 3); lean_dec(x_174); if (x_175 == 0) { @@ -9431,25 +9432,6 @@ return x_17; } } } -static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Elab_addAndCompilePartialRec___spec__2___closed__1() { -_start: -{ -lean_object* x_1; uint8_t x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; -x_1 = lean_box(0); -x_2 = 0; -x_3 = 0; -x_4 = 2; -x_5 = l___private_Lean_Elab_PreDefinition_Basic_0__Lean_Elab_getLevelParamsPreDecls___closed__4; -x_6 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_6, 0, x_1); -lean_ctor_set(x_6, 1, x_5); -lean_ctor_set_uint8(x_6, sizeof(void*)*2, x_2); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 1, x_3); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 2, x_4); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 3, x_3); -return x_6; -} -} LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_addAndCompilePartialRec___spec__2(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { _start: { @@ -9485,7 +9467,7 @@ lean_closure_set(x_16, 1, x_1); x_17 = lean_replace_expr(x_16, x_12); lean_dec(x_12); lean_dec(x_16); -x_18 = l_Array_mapMUnsafe_map___at_Lean_Elab_addAndCompilePartialRec___spec__2___closed__1; +x_18 = l_Lean_Elab_instInhabitedPreDefinition___closed__2; lean_ctor_set(x_7, 5, x_17); lean_ctor_set(x_7, 3, x_15); lean_ctor_set(x_7, 2, x_18); @@ -9523,7 +9505,7 @@ lean_closure_set(x_32, 1, x_1); x_33 = lean_replace_expr(x_32, x_28); lean_dec(x_28); lean_dec(x_32); -x_34 = l_Array_mapMUnsafe_map___at_Lean_Elab_addAndCompilePartialRec___spec__2___closed__1; +x_34 = l_Lean_Elab_instInhabitedPreDefinition___closed__2; x_35 = lean_alloc_ctor(0, 7, 1); lean_ctor_set(x_35, 0, x_23); lean_ctor_set(x_35, 1, x_25); @@ -9983,7 +9965,7 @@ else { lean_object* x_5; uint8_t x_6; x_5 = l_Lean_Expr_constName_x21(x_2); -x_6 = l_Array_contains___at_Lean_findField_x3f___spec__1(x_1, x_5); +x_6 = l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(x_1, x_5); lean_dec(x_5); return x_6; } @@ -10072,7 +10054,7 @@ else lean_object* x_12; uint8_t x_13; x_12 = l_Lean_Expr_constName_x21(x_8); lean_dec(x_8); -x_13 = l_Array_contains___at_Lean_findField_x3f___spec__1(x_1, x_12); +x_13 = l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(x_1, x_12); lean_dec(x_12); if (x_13 == 0) { @@ -13518,8 +13500,6 @@ l_Lean_Elab_addAndCompileUnsafe___boxed__const__1 = _init_l_Lean_Elab_addAndComp lean_mark_persistent(l_Lean_Elab_addAndCompileUnsafe___boxed__const__1); l_Array_mapMUnsafe_map___at_Lean_Elab_addAndCompilePartialRec___spec__2___lambda__1___closed__1 = _init_l_Array_mapMUnsafe_map___at_Lean_Elab_addAndCompilePartialRec___spec__2___lambda__1___closed__1(); lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Elab_addAndCompilePartialRec___spec__2___lambda__1___closed__1); -l_Array_mapMUnsafe_map___at_Lean_Elab_addAndCompilePartialRec___spec__2___closed__1 = _init_l_Array_mapMUnsafe_map___at_Lean_Elab_addAndCompilePartialRec___spec__2___closed__1(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Elab_addAndCompilePartialRec___spec__2___closed__1); l_Lean_Elab_ensureNoRecFn___lambda__1___closed__1 = _init_l_Lean_Elab_ensureNoRecFn___lambda__1___closed__1(); lean_mark_persistent(l_Lean_Elab_ensureNoRecFn___lambda__1___closed__1); l_Lean_Elab_ensureNoRecFn___lambda__1___closed__2 = _init_l_Lean_Elab_ensureNoRecFn___lambda__1___closed__2(); diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/Main.c b/stage0/stdlib/Lean/Elab/PreDefinition/Main.c index 1718b6022d6f..8bad5ff25bbd 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/Main.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/Main.c @@ -12911,7 +12911,7 @@ lean_ctor_set(x_18, 1, x_16); lean_ctor_set(x_18, 2, x_17); x_19 = lean_ctor_get(x_14, 2); lean_inc(x_19); -x_20 = lean_ctor_get_uint8(x_19, sizeof(void*)*2 + 3); +x_20 = lean_ctor_get_uint8(x_19, sizeof(void*)*3 + 3); lean_dec(x_19); x_21 = lean_alloc_ctor(0, 1, 1); lean_ctor_set(x_21, 0, x_18); @@ -16700,7 +16700,7 @@ x_5 = lean_array_uget(x_1, x_2); x_6 = lean_ctor_get(x_5, 2); lean_inc(x_6); lean_dec(x_5); -x_7 = lean_ctor_get_uint8(x_6, sizeof(void*)*2 + 3); +x_7 = lean_ctor_get_uint8(x_6, sizeof(void*)*3 + 3); lean_dec(x_6); if (x_7 == 0) { @@ -18613,7 +18613,7 @@ if (lean_obj_tag(x_28) == 0) lean_object* x_29; uint8_t x_30; x_29 = lean_ctor_get(x_25, 2); lean_inc(x_29); -x_30 = lean_ctor_get_uint8(x_29, sizeof(void*)*2 + 1); +x_30 = lean_ctor_get_uint8(x_29, sizeof(void*)*3 + 1); lean_dec(x_29); if (x_30 == 0) { diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/MkInhabitant.c b/stage0/stdlib/Lean/Elab/PreDefinition/MkInhabitant.c index 23b57b1faf5d..84876af096dc 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/MkInhabitant.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/MkInhabitant.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Lean.Elab.PreDefinition.MkInhabitant -// Imports: Lean.Meta.AppBuilder +// Imports: Lean.Meta.AppBuilder Lean.PrettyPrinter #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -13,49 +13,404 @@ #ifdef __cplusplus extern "C" { #endif +lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); +static lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__3; +static lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__5; +extern lean_object* l_Lean_maxRecDepthErrorMessage; uint8_t l_Lean_Exception_isInterrupt(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_Array_toSubarray___rarg(lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_mkAppB(lean_object*, lean_object*, lean_object*); +lean_object* lean_array_push(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_mkInhabitantFor___lambda__1___closed__9; +LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___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_array_fget(lean_object*, lean_object*); +lean_object* l_Lean_Meta_forallTelescope___at_Lean_Meta_mapForallTelescope_x27___spec__1___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_stringToMessageData(lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_findAssumption_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__6; +LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_mkInhabitantFor___lambda__1___closed__16; +static lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___closed__1; lean_object* l_Lean_throwError___at_Lean_Expr_abstractRangeM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_findAssumption_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkFnInhabitant_x3f_loop(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_outOfBounds___rarg(lean_object*); -static lean_object* l_Lean_Elab_mkInhabitantFor___closed__4; -LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_findAssumption_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -extern lean_object* l_Lean_instInhabitedExpr; -static lean_object* l_Lean_Elab_mkInhabitantFor___closed__1; +static lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__6; +lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withLetDeclImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances(lean_object*); +static lean_object* l_Lean_Elab_mkInhabitantFor___lambda__1___closed__5; +static lean_object* l_Lean_Elab_mkInhabitantFor___lambda__1___closed__11; +static lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__4; +LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_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_EXPORT lean_object* l_Lean_Meta_withLetDecl___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_MessageData_ofFormat(lean_object*); +static lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__1; +lean_object* l_Lean_Meta_getLevel(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_mkInhabitantFor___lambda__1___closed__6; +static lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__5; +static lean_object* l_Lean_Elab_mkInhabitantFor___lambda__1___closed__3; +lean_object* l_Lean_Meta_whnfEasyCases___at_Lean_Meta_whnfCore_go___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_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__2; +lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___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_MkInhabitant_0__Lean_Elab_mkInhabitant_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkFnInhabitant_x3f_loop___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__1; +static lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances___rarg___closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___lambda__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkDefault(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_MessageData_ofConstName(lean_object*); +lean_object* l_Array_append___rarg(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_mkInhabitantFor___lambda__1___closed__10; +LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___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_mkInhabitantFor___lambda__1___closed__4; +static lean_object* l_Lean_Elab_mkInhabitantFor___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_mkInhabitantFor(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*); +static lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__4; uint8_t lean_nat_dec_eq(lean_object*, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_findAssumption_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_mkInhabitantFor___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); +lean_object* l_Lean_indentExpr(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitant_x3f(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkFnInhabitant_x3f(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_findAssumption_x3f___closed__1; +lean_object* l_Lean_Meta_unfoldDefinition_x3f(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* lean_nat_sub(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_findAssumption_x3f___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_Array_ofSubarray___rarg(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go(lean_object*); +static lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__2; lean_object* lean_array_mk(lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkFnInhabitant_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -size_t lean_usize_add(size_t, size_t); -lean_object* lean_array_uget(lean_object*, size_t); -size_t lean_array_size(lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_findAssumption_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*); +static lean_object* l_Lean_Elab_mkInhabitantFor___lambda__1___closed__14; +static lean_object* l_Lean_Elab_mkInhabitantFor___lambda__1___closed__15; +LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -uint8_t lean_usize_dec_lt(size_t, size_t); lean_object* l_Lean_Meta_mkLambdaFVars(lean_object*, lean_object*, uint8_t, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_mkInhabitantFor___closed__3; +lean_object* lean_nat_add(lean_object*, lean_object*); uint8_t l_Lean_Exception_isRuntime(lean_object*); +static lean_object* l_Lean_Elab_mkInhabitantFor___lambda__1___closed__12; +uint8_t l_Lean_Expr_isForall(lean_object*); +static lean_object* l_Lean_Elab_mkInhabitantFor___lambda__1___closed__2; lean_object* l_Lean_Meta_mkOfNonempty(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_mkInhabitantFor___closed__2; +LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___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___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofName(lean_object*); +static lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__3; +static lean_object* l_Lean_Elab_mkInhabitantFor___lambda__1___closed__13; +LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_mkInhabitantFor___lambda__1___closed__7; +static lean_object* l_Lean_Elab_mkInhabitantFor___lambda__1___closed__8; +LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___spec__1(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___spec__1___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_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l___private_Lean_Meta_Basic_0__Lean_Meta_withLetDeclImp___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_11) == 0) +{ +uint8_t x_12; +x_12 = !lean_is_exclusive(x_11); +if (x_12 == 0) +{ +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_withLetDecl___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___spec__1(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLetDecl___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___spec__1___rarg___boxed), 10, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___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; lean_object* x_14; +x_11 = lean_unsigned_to_nat(1u); +x_12 = lean_nat_add(x_1, x_11); +x_13 = lean_array_push(x_2, x_5); +x_14 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg(x_3, x_4, x_12, x_13, x_6, x_7, x_8, x_9, x_10); +return x_14; +} +} +static lean_object* _init_l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Inhabited", 9, 9); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___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_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mk", 2, 2); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__1; +x_2 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__3; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("inst", 4, 4); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___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_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__5; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___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; uint8_t x_11; +x_10 = lean_array_get_size(x_1); +x_11 = lean_nat_dec_lt(x_3, x_10); +lean_dec(x_10); +if (x_11 == 0) +{ +lean_object* x_12; +lean_dec(x_3); +lean_dec(x_1); +x_12 = lean_apply_6(x_2, x_4, x_5, x_6, x_7, x_8, x_9); +return x_12; +} +else +{ +lean_object* x_13; lean_object* x_14; +x_13 = lean_array_fget(x_1, x_3); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_13); +x_14 = lean_infer_type(x_13, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_14) == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_15); +x_17 = l_Lean_Meta_getLevel(x_15, x_5, x_6, x_7, x_8, x_16); +if (lean_obj_tag(x_17) == 0) +{ +lean_object* x_18; lean_object* x_19; 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; uint8_t x_30; lean_object* x_31; +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); +lean_dec(x_17); +x_20 = lean_box(0); +x_21 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_21, 0, x_18); +lean_ctor_set(x_21, 1, x_20); +x_22 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__2; +lean_inc(x_21); +x_23 = l_Lean_Expr_const___override(x_22, x_21); +lean_inc(x_15); +x_24 = l_Lean_Expr_app___override(x_23, x_15); +x_25 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__4; +x_26 = l_Lean_Expr_const___override(x_25, x_21); +x_27 = l_Lean_mkAppB(x_26, x_15, x_13); +x_28 = lean_alloc_closure((void*)(l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___lambda__1___boxed), 10, 4); +lean_closure_set(x_28, 0, x_3); +lean_closure_set(x_28, 1, x_4); +lean_closure_set(x_28, 2, x_1); +lean_closure_set(x_28, 3, x_2); +x_29 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__6; +x_30 = 0; +x_31 = l_Lean_Meta_withLetDecl___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___spec__1___rarg(x_29, x_24, x_27, x_28, x_30, x_5, x_6, x_7, x_8, x_19); +return x_31; +} +else +{ +uint8_t x_32; +lean_dec(x_15); +lean_dec(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); +lean_dec(x_1); +x_32 = !lean_is_exclusive(x_17); +if (x_32 == 0) +{ +return x_17; +} +else +{ +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_17, 0); +x_34 = lean_ctor_get(x_17, 1); +lean_inc(x_34); +lean_inc(x_33); +lean_dec(x_17); +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +return x_35; +} +} +} +else +{ +uint8_t x_36; +lean_dec(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); +lean_dec(x_1); +x_36 = !lean_is_exclusive(x_14); +if (x_36 == 0) +{ +return x_14; +} +else +{ +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_14, 0); +x_38 = lean_ctor_get(x_14, 1); +lean_inc(x_38); +lean_inc(x_37); +lean_dec(x_14); +x_39 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_39, 0, x_37); +lean_ctor_set(x_39, 1, x_38); +return x_39; +} +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg), 9, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, 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_5); +lean_dec(x_5); +x_12 = l_Lean_Meta_withLetDecl___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___spec__1___rarg(x_1, x_2, x_3, x_4, x_11, x_6, x_7, x_8, x_9, x_10); +return x_12; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_1); +return x_11; +} +} +static lean_object* _init_l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances___rarg___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_array_mk(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances___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; +x_8 = lean_unsigned_to_nat(0u); +x_9 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances___rarg___closed__1; +x_10 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg(x_1, x_2, x_8, x_9, x_3, x_4, x_5, x_6, x_7); +return x_10; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances___rarg), 7, 0); +return x_2; +} +} LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitant_x3f(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: { @@ -200,559 +555,297 @@ x_9 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitant return x_9; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_findAssumption_x3f___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +static lean_object* _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__1() { _start: { -uint8_t x_12; -x_12 = lean_usize_dec_lt(x_5, x_4); -if (x_12 == 0) -{ -lean_object* x_13; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_2); -lean_dec(x_1); -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_6); -lean_ctor_set(x_13, 1, x_11); -return x_13; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("runtime", 7, 7); +return x_1; } -else +} +static lean_object* _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__2() { +_start: { -lean_object* x_14; lean_object* x_15; -lean_dec(x_6); -x_14 = lean_array_uget(x_3, x_5); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_14); -x_15 = lean_infer_type(x_14, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_15) == 0) +lean_object* x_1; +x_1 = lean_mk_string_unchecked("maxRecDepth", 11, 11); +return x_1; +} +} +static lean_object* _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__3() { +_start: { -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_15, 0); -lean_inc(x_16); -x_17 = lean_ctor_get(x_15, 1); -lean_inc(x_17); -lean_dec(x_15); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_1); -x_18 = l_Lean_Meta_isExprDefEq(x_16, x_1, x_7, x_8, x_9, x_10, x_17); -if (lean_obj_tag(x_18) == 0) +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__1; +x_2 = l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__2; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__4() { +_start: { -lean_object* x_19; uint8_t x_20; -x_19 = lean_ctor_get(x_18, 0); -lean_inc(x_19); -x_20 = lean_unbox(x_19); -lean_dec(x_19); -if (x_20 == 0) +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_maxRecDepthErrorMessage; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__5() { +_start: { -lean_object* x_21; size_t x_22; size_t x_23; -lean_dec(x_14); -x_21 = lean_ctor_get(x_18, 1); -lean_inc(x_21); -lean_dec(x_18); -x_22 = 1; -x_23 = lean_usize_add(x_5, x_22); -lean_inc(x_2); +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__4; +x_2 = l_Lean_MessageData_ofFormat(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__6() { +_start: { -size_t _tmp_4 = x_23; -lean_object* _tmp_5 = x_2; -lean_object* _tmp_10 = x_21; -x_5 = _tmp_4; -x_6 = _tmp_5; -x_11 = _tmp_10; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__3; +x_2 = l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__5; +x_3 = lean_alloc_ctor(8, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; } -goto _start; } -else +LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___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: { -uint8_t x_25; -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_25 = !lean_is_exclusive(x_18); -if (x_25 == 0) -{ -lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_26 = lean_ctor_get(x_18, 0); -lean_dec(x_26); -x_27 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_27, 0, x_14); -x_28 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_28, 0, x_27); -x_29 = lean_box(0); -x_30 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_30, 0, x_28); -lean_ctor_set(x_30, 1, x_29); -lean_ctor_set(x_18, 0, x_30); -return x_18; -} -else -{ -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_31 = lean_ctor_get(x_18, 1); -lean_inc(x_31); -lean_dec(x_18); -x_32 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_32, 0, x_14); -x_33 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_33, 0, x_32); -x_34 = lean_box(0); -x_35 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_35, 0, x_33); -lean_ctor_set(x_35, 1, x_34); -x_36 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_36, 0, x_35); -lean_ctor_set(x_36, 1, x_31); -return x_36; -} -} -} -else -{ -uint8_t x_37; -lean_dec(x_14); -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_37 = !lean_is_exclusive(x_18); -if (x_37 == 0) -{ -return x_18; -} -else -{ -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_18, 0); -x_39 = lean_ctor_get(x_18, 1); -lean_inc(x_39); -lean_inc(x_38); -lean_dec(x_18); -x_40 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_40, 0, x_38); -lean_ctor_set(x_40, 1, x_39); -return x_40; -} +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__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_alloc_ctor(1, 2, 0); +lean_ctor_set(x_9, 0, x_8); +lean_ctor_set(x_9, 1, x_6); +return x_9; } } -else -{ -uint8_t x_41; -lean_dec(x_14); -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_41 = !lean_is_exclusive(x_15); -if (x_41 == 0) -{ -return x_15; -} -else +LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___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_object* x_11) { +_start: { -lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_ctor_get(x_15, 0); -x_43 = lean_ctor_get(x_15, 1); -lean_inc(x_43); -lean_inc(x_42); -lean_dec(x_15); -x_44 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_44, 0, x_42); -lean_ctor_set(x_44, 1, x_43); -return x_44; -} -} -} +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = l_Array_append___rarg(x_1, x_2); +x_13 = l_Array_append___rarg(x_3, x_6); +x_14 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f(x_12, x_13, x_4, x_5, x_7, x_8, x_9, x_10, x_11); +return x_14; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_findAssumption_x3f___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___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_8; -x_8 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_8, 0, x_1); -lean_ctor_set(x_8, 1, x_7); -return x_8; +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_box(x_3); +lean_inc(x_4); +x_12 = lean_alloc_closure((void*)(l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___lambda__1___boxed), 11, 5); +lean_closure_set(x_12, 0, x_1); +lean_closure_set(x_12, 1, x_4); +lean_closure_set(x_12, 2, x_2); +lean_closure_set(x_12, 3, x_5); +lean_closure_set(x_12, 4, x_11); +x_13 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances___rarg(x_4, x_12, x_6, x_7, x_8, x_9, x_10); +return x_13; } } -static lean_object* _init_l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_findAssumption_x3f___closed__1() { +static lean_object* _init_l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___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); +uint8_t x_1; uint8_t x_2; lean_object* x_3; +x_1 = 1; +x_2 = 2; +x_3 = lean_alloc_ctor(0, 0, 5); +lean_ctor_set_uint8(x_3, 0, x_1); +lean_ctor_set_uint8(x_3, 1, x_1); +lean_ctor_set_uint8(x_3, 2, x_2); +lean_ctor_set_uint8(x_3, 3, x_1); +lean_ctor_set_uint8(x_3, 4, x_1); return x_3; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_findAssumption_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_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_8; size_t x_9; size_t x_10; lean_object* x_11; lean_object* x_12; -x_8 = lean_box(0); -x_9 = lean_array_size(x_1); -x_10 = 0; -x_11 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_findAssumption_x3f___closed__1; -x_12 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_findAssumption_x3f___spec__1(x_2, x_11, x_1, x_9, x_10, x_11, x_3, x_4, x_5, x_6, x_7); -if (lean_obj_tag(x_12) == 0) -{ -lean_object* x_13; lean_object* x_14; -x_13 = lean_ctor_get(x_12, 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; uint8_t x_21; lean_object* x_22; uint8_t x_23; uint8_t x_24; +x_10 = lean_ctor_get(x_7, 0); +lean_inc(x_10); +x_11 = lean_ctor_get(x_7, 1); +lean_inc(x_11); +x_12 = lean_ctor_get(x_7, 2); +lean_inc(x_12); +x_13 = lean_ctor_get(x_7, 3); lean_inc(x_13); -x_14 = lean_ctor_get(x_13, 0); +x_14 = lean_ctor_get(x_7, 4); lean_inc(x_14); -lean_dec(x_13); -if (lean_obj_tag(x_14) == 0) -{ -uint8_t x_15; -x_15 = !lean_is_exclusive(x_12); -if (x_15 == 0) -{ -lean_object* x_16; -x_16 = lean_ctor_get(x_12, 0); -lean_dec(x_16); -lean_ctor_set(x_12, 0, x_8); -return x_12; -} -else -{ -lean_object* x_17; lean_object* x_18; -x_17 = lean_ctor_get(x_12, 1); +x_15 = lean_ctor_get(x_7, 5); +lean_inc(x_15); +x_16 = lean_ctor_get(x_7, 6); +lean_inc(x_16); +x_17 = lean_ctor_get(x_7, 7); lean_inc(x_17); -lean_dec(x_12); -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 -{ -uint8_t x_19; -x_19 = !lean_is_exclusive(x_12); -if (x_19 == 0) -{ -lean_object* x_20; lean_object* x_21; -x_20 = lean_ctor_get(x_12, 0); -lean_dec(x_20); -x_21 = lean_ctor_get(x_14, 0); -lean_inc(x_21); -lean_dec(x_14); -lean_ctor_set(x_12, 0, x_21); -return x_12; -} -else -{ -lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_22 = lean_ctor_get(x_12, 1); +x_18 = lean_ctor_get(x_7, 8); +lean_inc(x_18); +x_19 = lean_ctor_get(x_7, 9); +lean_inc(x_19); +x_20 = lean_ctor_get(x_7, 10); +lean_inc(x_20); +x_21 = lean_ctor_get_uint8(x_7, sizeof(void*)*12); +x_22 = lean_ctor_get(x_7, 11); lean_inc(x_22); -lean_dec(x_12); -x_23 = lean_ctor_get(x_14, 0); -lean_inc(x_23); -lean_dec(x_14); -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 +x_23 = lean_ctor_get_uint8(x_7, sizeof(void*)*12 + 1); +x_24 = lean_nat_dec_eq(x_13, x_14); +if (x_24 == 0) { uint8_t x_25; -x_25 = !lean_is_exclusive(x_12); +x_25 = !lean_is_exclusive(x_7); if (x_25 == 0) { -return x_12; -} -else -{ -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_12, 0); -x_27 = lean_ctor_get(x_12, 1); -lean_inc(x_27); -lean_inc(x_26); -lean_dec(x_12); -x_28 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_28, 0, x_26); -lean_ctor_set(x_28, 1, x_27); -return x_28; -} -} -} -} -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_findAssumption_x3f___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -size_t x_12; size_t x_13; lean_object* x_14; -x_12 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_13 = lean_unbox_usize(x_5); -lean_dec(x_5); -x_14 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_findAssumption_x3f___spec__1(x_1, x_2, x_3, x_12, x_13, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_3); -return x_14; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_findAssumption_x3f___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; -x_8 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_findAssumption_x3f___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_8; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_findAssumption_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) { -_start: -{ -lean_object* x_8; -x_8 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_findAssumption_x3f(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_PreDefinition_MkInhabitant_0__Lean_Elab_mkFnInhabitant_x3f_loop(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; uint8_t x_11; -x_10 = lean_unsigned_to_nat(0u); -x_11 = lean_nat_dec_eq(x_3, x_10); -if (x_11 == 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; +x_26 = lean_ctor_get(x_7, 11); +lean_dec(x_26); +x_27 = lean_ctor_get(x_7, 10); +lean_dec(x_27); +x_28 = lean_ctor_get(x_7, 9); +lean_dec(x_28); +x_29 = lean_ctor_get(x_7, 8); +lean_dec(x_29); +x_30 = lean_ctor_get(x_7, 7); +lean_dec(x_30); +x_31 = lean_ctor_get(x_7, 6); +lean_dec(x_31); +x_32 = lean_ctor_get(x_7, 5); +lean_dec(x_32); +x_33 = lean_ctor_get(x_7, 4); +lean_dec(x_33); +x_34 = lean_ctor_get(x_7, 3); +lean_dec(x_34); +x_35 = lean_ctor_get(x_7, 2); +lean_dec(x_35); +x_36 = lean_ctor_get(x_7, 1); +lean_dec(x_36); +x_37 = lean_ctor_get(x_7, 0); +lean_dec(x_37); +x_38 = lean_unsigned_to_nat(1u); +x_39 = lean_nat_add(x_13, x_38); +lean_dec(x_13); +lean_ctor_set(x_7, 3, x_39); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_3); +x_40 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitant_x3f(x_3, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_40) == 0) { -lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; lean_object* x_16; -x_12 = lean_unsigned_to_nat(1u); -x_13 = lean_nat_sub(x_3, x_12); -lean_dec(x_3); -x_14 = lean_array_get_size(x_1); -x_15 = lean_nat_dec_lt(x_13, x_14); -lean_dec(x_14); -x_16 = lean_box(0); -if (x_15 == 0) +lean_object* x_41; +x_41 = lean_ctor_get(x_40, 0); +lean_inc(x_41); +if (lean_obj_tag(x_41) == 0) { -lean_object* x_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; lean_object* x_24; -x_17 = l_Lean_instInhabitedExpr; -x_18 = l_outOfBounds___rarg(x_17); -x_19 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_19, 0, x_18); -lean_ctor_set(x_19, 1, x_16); -x_20 = lean_array_mk(x_19); -x_21 = 0; -x_22 = 1; -x_23 = 1; -x_24 = l_Lean_Meta_mkForallFVars(x_20, x_4, x_21, x_22, x_23, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_24) == 0) -{ -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_24, 0); -lean_inc(x_25); -x_26 = lean_ctor_get(x_24, 1); -lean_inc(x_26); -lean_dec(x_24); +lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_42 = lean_ctor_get(x_40, 1); +lean_inc(x_42); +lean_dec(x_40); +x_43 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___closed__1; lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -lean_inc(x_25); -x_27 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitant_x3f(x_25, x_2, x_5, x_6, x_7, x_8, x_26); -if (lean_obj_tag(x_27) == 0) +x_44 = l_Lean_Meta_whnfEasyCases___at_Lean_Meta_whnfCore_go___spec__2(x_43, x_3, x_43, x_5, x_6, x_7, x_8, x_42); +if (lean_obj_tag(x_44) == 0) { -lean_object* x_28; -x_28 = lean_ctor_get(x_27, 0); -lean_inc(x_28); -if (lean_obj_tag(x_28) == 0) +lean_object* x_45; lean_object* x_46; uint8_t x_47; +x_45 = lean_ctor_get(x_44, 0); +lean_inc(x_45); +x_46 = lean_ctor_get(x_44, 1); +lean_inc(x_46); +lean_dec(x_44); +x_47 = l_Lean_Expr_isForall(x_45); +if (x_47 == 0) { -lean_object* x_29; -x_29 = lean_ctor_get(x_27, 1); -lean_inc(x_29); -lean_dec(x_27); -x_3 = x_13; -x_4 = x_25; -x_9 = x_29; -goto _start; -} -else +lean_object* x_48; +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_48 = l_Lean_Meta_unfoldDefinition_x3f(x_45, x_5, x_6, x_7, x_8, x_46); +if (lean_obj_tag(x_48) == 0) { -lean_object* x_31; uint8_t x_32; -lean_dec(x_25); -x_31 = lean_ctor_get(x_27, 1); -lean_inc(x_31); -lean_dec(x_27); -x_32 = !lean_is_exclusive(x_28); -if (x_32 == 0) +lean_object* x_49; +x_49 = lean_ctor_get(x_48, 0); +lean_inc(x_49); +if (lean_obj_tag(x_49) == 0) { -lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_33 = lean_ctor_get(x_28, 0); -x_34 = l_Array_toSubarray___rarg(x_1, x_10, x_13); -x_35 = l_Array_ofSubarray___rarg(x_34); -lean_dec(x_34); -x_36 = l_Lean_Meta_mkLambdaFVars(x_35, x_33, x_21, x_22, x_21, x_23, x_5, x_6, x_7, x_8, x_31); -lean_dec(x_8); +uint8_t x_50; lean_dec(x_7); +lean_dec(x_8); lean_dec(x_6); lean_dec(x_5); -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; -x_38 = lean_ctor_get(x_36, 0); -lean_ctor_set(x_28, 0, x_38); -lean_ctor_set(x_36, 0, x_28); -return x_36; -} -else -{ -lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_39 = lean_ctor_get(x_36, 0); -x_40 = lean_ctor_get(x_36, 1); -lean_inc(x_40); -lean_inc(x_39); -lean_dec(x_36); -lean_ctor_set(x_28, 0, x_39); -x_41 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_41, 0, x_28); -lean_ctor_set(x_41, 1, x_40); -return x_41; -} -} -else -{ -uint8_t x_42; -lean_free_object(x_28); -x_42 = !lean_is_exclusive(x_36); -if (x_42 == 0) -{ -return x_36; -} -else +lean_dec(x_2); +lean_dec(x_1); +x_50 = !lean_is_exclusive(x_48); +if (x_50 == 0) { -lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_43 = lean_ctor_get(x_36, 0); -x_44 = lean_ctor_get(x_36, 1); -lean_inc(x_44); -lean_inc(x_43); -lean_dec(x_36); -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_51; lean_object* x_52; +x_51 = lean_ctor_get(x_48, 0); +lean_dec(x_51); +x_52 = lean_box(0); +lean_ctor_set(x_48, 0, x_52); +return x_48; } else { -lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_46 = lean_ctor_get(x_28, 0); -lean_inc(x_46); -lean_dec(x_28); -x_47 = l_Array_toSubarray___rarg(x_1, x_10, x_13); -x_48 = l_Array_ofSubarray___rarg(x_47); -lean_dec(x_47); -x_49 = l_Lean_Meta_mkLambdaFVars(x_48, x_46, x_21, x_22, x_21, x_23, x_5, x_6, x_7, x_8, x_31); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -if (lean_obj_tag(x_49) == 0) -{ -lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; -x_50 = lean_ctor_get(x_49, 0); -lean_inc(x_50); -x_51 = lean_ctor_get(x_49, 1); -lean_inc(x_51); -if (lean_is_exclusive(x_49)) { - lean_ctor_release(x_49, 0); - lean_ctor_release(x_49, 1); - x_52 = x_49; -} else { - lean_dec_ref(x_49); - x_52 = lean_box(0); -} -x_53 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_53, 0, x_50); -if (lean_is_scalar(x_52)) { - x_54 = lean_alloc_ctor(0, 2, 0); -} else { - x_54 = x_52; +lean_object* x_53; lean_object* x_54; lean_object* x_55; +x_53 = lean_ctor_get(x_48, 1); +lean_inc(x_53); +lean_dec(x_48); +x_54 = lean_box(0); +x_55 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_55, 0, x_54); +lean_ctor_set(x_55, 1, x_53); +return x_55; } -lean_ctor_set(x_54, 0, x_53); -lean_ctor_set(x_54, 1, x_51); -return x_54; } else { -lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; -x_55 = lean_ctor_get(x_49, 0); -lean_inc(x_55); -x_56 = lean_ctor_get(x_49, 1); +lean_object* x_56; lean_object* x_57; +x_56 = lean_ctor_get(x_48, 1); lean_inc(x_56); -if (lean_is_exclusive(x_49)) { - lean_ctor_release(x_49, 0); - lean_ctor_release(x_49, 1); - x_57 = x_49; -} else { - lean_dec_ref(x_49); - 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_dec(x_48); +x_57 = lean_ctor_get(x_49, 0); +lean_inc(x_57); +lean_dec(x_49); +x_3 = x_57; +x_9 = x_56; +goto _start; } } else { uint8_t x_59; -lean_dec(x_25); -lean_dec(x_13); -lean_dec(x_8); lean_dec(x_7); +lean_dec(x_8); lean_dec(x_6); lean_dec(x_5); +lean_dec(x_2); lean_dec(x_1); -x_59 = !lean_is_exclusive(x_27); +x_59 = !lean_is_exclusive(x_48); if (x_59 == 0) { -return x_27; +return x_48; } else { lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_60 = lean_ctor_get(x_27, 0); -x_61 = lean_ctor_get(x_27, 1); +x_60 = lean_ctor_get(x_48, 0); +x_61 = lean_ctor_get(x_48, 1); lean_inc(x_61); lean_inc(x_60); -lean_dec(x_27); +lean_dec(x_48); x_62 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_62, 0, x_60); lean_ctor_set(x_62, 1, x_61); @@ -762,1131 +855,929 @@ return x_62; } else { -uint8_t x_63; -lean_dec(x_13); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_1); -x_63 = !lean_is_exclusive(x_24); -if (x_63 == 0) -{ -return x_24; -} -else -{ -lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_64 = lean_ctor_get(x_24, 0); -x_65 = lean_ctor_get(x_24, 1); -lean_inc(x_65); -lean_inc(x_64); -lean_dec(x_24); -x_66 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_66, 0, x_64); -lean_ctor_set(x_66, 1, x_65); +lean_object* x_63; lean_object* x_64; uint8_t x_65; lean_object* x_66; +x_63 = lean_box(x_4); +x_64 = lean_alloc_closure((void*)(l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___lambda__2___boxed), 10, 3); +lean_closure_set(x_64, 0, x_1); +lean_closure_set(x_64, 1, x_2); +lean_closure_set(x_64, 2, x_63); +x_65 = 0; +x_66 = l_Lean_Meta_forallTelescope___at_Lean_Meta_mapForallTelescope_x27___spec__1___rarg(x_45, x_64, x_65, x_5, x_6, x_7, x_8, x_46); return x_66; } } -} -else -{ -lean_object* x_67; lean_object* x_68; lean_object* x_69; uint8_t x_70; uint8_t x_71; uint8_t x_72; lean_object* x_73; -x_67 = lean_array_fget(x_1, x_13); -x_68 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_68, 0, x_67); -lean_ctor_set(x_68, 1, x_16); -x_69 = lean_array_mk(x_68); -x_70 = 0; -x_71 = 1; -x_72 = 1; -x_73 = l_Lean_Meta_mkForallFVars(x_69, x_4, x_70, x_71, x_72, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_73) == 0) -{ -lean_object* x_74; lean_object* x_75; lean_object* 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); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_74); -x_76 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitant_x3f(x_74, x_2, x_5, x_6, x_7, x_8, x_75); -if (lean_obj_tag(x_76) == 0) -{ -lean_object* x_77; -x_77 = lean_ctor_get(x_76, 0); -lean_inc(x_77); -if (lean_obj_tag(x_77) == 0) -{ -lean_object* x_78; -x_78 = lean_ctor_get(x_76, 1); -lean_inc(x_78); -lean_dec(x_76); -x_3 = x_13; -x_4 = x_74; -x_9 = x_78; -goto _start; -} else { -lean_object* x_80; uint8_t x_81; -lean_dec(x_74); -x_80 = lean_ctor_get(x_76, 1); -lean_inc(x_80); -lean_dec(x_76); -x_81 = !lean_is_exclusive(x_77); -if (x_81 == 0) -{ -lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; -x_82 = lean_ctor_get(x_77, 0); -x_83 = l_Array_toSubarray___rarg(x_1, x_10, x_13); -x_84 = l_Array_ofSubarray___rarg(x_83); -lean_dec(x_83); -x_85 = l_Lean_Meta_mkLambdaFVars(x_84, x_82, x_70, x_71, x_70, x_72, x_5, x_6, x_7, x_8, x_80); -lean_dec(x_8); +uint8_t x_67; lean_dec(x_7); +lean_dec(x_8); lean_dec(x_6); lean_dec(x_5); -if (lean_obj_tag(x_85) == 0) -{ -uint8_t x_86; -x_86 = !lean_is_exclusive(x_85); -if (x_86 == 0) +lean_dec(x_2); +lean_dec(x_1); +x_67 = !lean_is_exclusive(x_44); +if (x_67 == 0) { -lean_object* x_87; -x_87 = lean_ctor_get(x_85, 0); -lean_ctor_set(x_77, 0, x_87); -lean_ctor_set(x_85, 0, x_77); -return x_85; +return x_44; } else { -lean_object* x_88; lean_object* x_89; lean_object* x_90; -x_88 = lean_ctor_get(x_85, 0); -x_89 = lean_ctor_get(x_85, 1); -lean_inc(x_89); -lean_inc(x_88); -lean_dec(x_85); -lean_ctor_set(x_77, 0, x_88); -x_90 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_90, 0, x_77); -lean_ctor_set(x_90, 1, x_89); -return x_90; +lean_object* x_68; lean_object* x_69; lean_object* x_70; +x_68 = lean_ctor_get(x_44, 0); +x_69 = lean_ctor_get(x_44, 1); +lean_inc(x_69); +lean_inc(x_68); +lean_dec(x_44); +x_70 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_70, 0, x_68); +lean_ctor_set(x_70, 1, x_69); +return x_70; } } -else -{ -uint8_t x_91; -lean_free_object(x_77); -x_91 = !lean_is_exclusive(x_85); -if (x_91 == 0) -{ -return x_85; } else { -lean_object* x_92; lean_object* x_93; lean_object* x_94; -x_92 = lean_ctor_get(x_85, 0); -x_93 = lean_ctor_get(x_85, 1); -lean_inc(x_93); -lean_inc(x_92); -lean_dec(x_85); -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 +lean_object* x_71; uint8_t x_72; +lean_dec(x_3); +x_71 = lean_ctor_get(x_40, 1); +lean_inc(x_71); +lean_dec(x_40); +x_72 = !lean_is_exclusive(x_41); +if (x_72 == 0) +{ +lean_object* x_73; uint8_t x_74; uint8_t x_75; uint8_t x_76; lean_object* x_77; +x_73 = lean_ctor_get(x_41, 0); +x_74 = 0; +x_75 = 1; +x_76 = 1; +x_77 = l_Lean_Meta_mkLambdaFVars(x_2, x_73, x_74, x_75, x_74, x_76, x_5, x_6, x_7, x_8, x_71); +if (lean_obj_tag(x_77) == 0) { -lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; -x_95 = lean_ctor_get(x_77, 0); -lean_inc(x_95); +lean_object* x_78; lean_object* x_79; lean_object* x_80; +x_78 = lean_ctor_get(x_77, 0); +lean_inc(x_78); +x_79 = lean_ctor_get(x_77, 1); +lean_inc(x_79); lean_dec(x_77); -x_96 = l_Array_toSubarray___rarg(x_1, x_10, x_13); -x_97 = l_Array_ofSubarray___rarg(x_96); -lean_dec(x_96); -x_98 = l_Lean_Meta_mkLambdaFVars(x_97, x_95, x_70, x_71, x_70, x_72, x_5, x_6, x_7, x_8, x_80); +x_80 = l_Lean_Meta_mkLambdaFVars(x_1, x_78, x_74, x_75, x_74, x_76, x_5, x_6, x_7, x_8, x_79); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -if (lean_obj_tag(x_98) == 0) +if (lean_obj_tag(x_80) == 0) { -lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; -x_99 = lean_ctor_get(x_98, 0); -lean_inc(x_99); -x_100 = lean_ctor_get(x_98, 1); -lean_inc(x_100); -if (lean_is_exclusive(x_98)) { - lean_ctor_release(x_98, 0); - lean_ctor_release(x_98, 1); - x_101 = x_98; -} else { - lean_dec_ref(x_98); - x_101 = lean_box(0); -} -x_102 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_102, 0, x_99); -if (lean_is_scalar(x_101)) { - x_103 = lean_alloc_ctor(0, 2, 0); -} else { - x_103 = x_101; -} -lean_ctor_set(x_103, 0, x_102); -lean_ctor_set(x_103, 1, x_100); -return x_103; +uint8_t x_81; +x_81 = !lean_is_exclusive(x_80); +if (x_81 == 0) +{ +lean_object* x_82; +x_82 = lean_ctor_get(x_80, 0); +lean_ctor_set(x_41, 0, x_82); +lean_ctor_set(x_80, 0, x_41); +return x_80; } else { -lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; -x_104 = lean_ctor_get(x_98, 0); -lean_inc(x_104); -x_105 = lean_ctor_get(x_98, 1); -lean_inc(x_105); -if (lean_is_exclusive(x_98)) { - lean_ctor_release(x_98, 0); - lean_ctor_release(x_98, 1); - x_106 = x_98; -} else { - lean_dec_ref(x_98); - 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_object* x_83; lean_object* x_84; lean_object* x_85; +x_83 = lean_ctor_get(x_80, 0); +x_84 = lean_ctor_get(x_80, 1); +lean_inc(x_84); +lean_inc(x_83); +lean_dec(x_80); +lean_ctor_set(x_41, 0, x_83); +x_85 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_85, 0, x_41); +lean_ctor_set(x_85, 1, x_84); +return x_85; } } -else -{ -uint8_t x_108; -lean_dec(x_74); -lean_dec(x_13); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_1); -x_108 = !lean_is_exclusive(x_76); -if (x_108 == 0) +else +{ +uint8_t x_86; +lean_free_object(x_41); +x_86 = !lean_is_exclusive(x_80); +if (x_86 == 0) { -return x_76; +return x_80; } else { -lean_object* x_109; lean_object* x_110; lean_object* x_111; -x_109 = lean_ctor_get(x_76, 0); -x_110 = lean_ctor_get(x_76, 1); -lean_inc(x_110); -lean_inc(x_109); -lean_dec(x_76); -x_111 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_111, 0, x_109); -lean_ctor_set(x_111, 1, x_110); -return x_111; +lean_object* x_87; lean_object* x_88; lean_object* x_89; +x_87 = lean_ctor_get(x_80, 0); +x_88 = lean_ctor_get(x_80, 1); +lean_inc(x_88); +lean_inc(x_87); +lean_dec(x_80); +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_112; -lean_dec(x_13); -lean_dec(x_8); +uint8_t x_90; +lean_free_object(x_41); lean_dec(x_7); +lean_dec(x_8); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_112 = !lean_is_exclusive(x_73); -if (x_112 == 0) +x_90 = !lean_is_exclusive(x_77); +if (x_90 == 0) { -return x_73; +return x_77; } else { -lean_object* x_113; lean_object* x_114; lean_object* x_115; -x_113 = lean_ctor_get(x_73, 0); -x_114 = lean_ctor_get(x_73, 1); -lean_inc(x_114); -lean_inc(x_113); -lean_dec(x_73); -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_91; lean_object* x_92; lean_object* x_93; +x_91 = lean_ctor_get(x_77, 0); +x_92 = lean_ctor_get(x_77, 1); +lean_inc(x_92); +lean_inc(x_91); +lean_dec(x_77); +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_116; -lean_dec(x_3); -lean_dec(x_1); -x_116 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitant_x3f(x_4, x_2, x_5, x_6, x_7, x_8, x_9); -return x_116; -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkFnInhabitant_x3f_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) { -_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_PreDefinition_MkInhabitant_0__Lean_Elab_mkFnInhabitant_x3f_loop(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___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkFnInhabitant_x3f(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: +lean_object* x_94; uint8_t x_95; uint8_t x_96; uint8_t x_97; lean_object* x_98; +x_94 = lean_ctor_get(x_41, 0); +lean_inc(x_94); +lean_dec(x_41); +x_95 = 0; +x_96 = 1; +x_97 = 1; +x_98 = l_Lean_Meta_mkLambdaFVars(x_2, x_94, x_95, x_96, x_95, x_97, x_5, x_6, x_7, x_8, x_71); +if (lean_obj_tag(x_98) == 0) { -lean_object* x_9; lean_object* x_10; -x_9 = lean_array_get_size(x_1); -x_10 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkFnInhabitant_x3f_loop(x_1, x_3, x_9, x_2, x_4, x_5, x_6, x_7, x_8); -return x_10; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkFnInhabitant_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_99; lean_object* x_100; lean_object* 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 = l_Lean_Meta_mkLambdaFVars(x_1, x_99, x_95, x_96, x_95, x_97, x_5, x_6, x_7, x_8, x_100); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +if (lean_obj_tag(x_101) == 0) { -uint8_t x_9; lean_object* x_10; -x_9 = lean_unbox(x_3); -lean_dec(x_3); -x_10 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkFnInhabitant_x3f(x_1, x_2, x_9, x_4, x_5, x_6, x_7, x_8); -return x_10; -} +lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; +x_102 = lean_ctor_get(x_101, 0); +lean_inc(x_102); +x_103 = lean_ctor_get(x_101, 1); +lean_inc(x_103); +if (lean_is_exclusive(x_101)) { + lean_ctor_release(x_101, 0); + lean_ctor_release(x_101, 1); + x_104 = x_101; +} else { + lean_dec_ref(x_101); + x_104 = lean_box(0); } -static lean_object* _init_l_Lean_Elab_mkInhabitantFor___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("failed to compile partial definition '", 38, 38); -return x_1; +x_105 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_105, 0, x_102); +if (lean_is_scalar(x_104)) { + x_106 = lean_alloc_ctor(0, 2, 0); +} else { + x_106 = x_104; } +lean_ctor_set(x_106, 0, x_105); +lean_ctor_set(x_106, 1, x_103); +return x_106; } -static lean_object* _init_l_Lean_Elab_mkInhabitantFor___closed__2() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_mkInhabitantFor___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; +x_107 = lean_ctor_get(x_101, 0); +lean_inc(x_107); +x_108 = lean_ctor_get(x_101, 1); +lean_inc(x_108); +if (lean_is_exclusive(x_101)) { + lean_ctor_release(x_101, 0); + lean_ctor_release(x_101, 1); + x_109 = x_101; +} else { + lean_dec_ref(x_101); + x_109 = lean_box(0); } +if (lean_is_scalar(x_109)) { + x_110 = lean_alloc_ctor(1, 2, 0); +} else { + x_110 = x_109; } -static lean_object* _init_l_Lean_Elab_mkInhabitantFor___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("', failed to show that type is inhabited and non empty", 54, 54); -return x_1; +lean_ctor_set(x_110, 0, x_107); +lean_ctor_set(x_110, 1, x_108); +return x_110; } } -static lean_object* _init_l_Lean_Elab_mkInhabitantFor___closed__4() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_mkInhabitantFor___closed__3; -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_dec(x_7); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_1); +x_111 = lean_ctor_get(x_98, 0); +lean_inc(x_111); +x_112 = lean_ctor_get(x_98, 1); +lean_inc(x_112); +if (lean_is_exclusive(x_98)) { + lean_ctor_release(x_98, 0); + lean_ctor_release(x_98, 1); + x_113 = x_98; +} else { + lean_dec_ref(x_98); + x_113 = lean_box(0); } -LEAN_EXPORT lean_object* l_Lean_Elab_mkInhabitantFor(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; lean_object* x_10; uint8_t x_98; lean_object* x_99; -x_98 = 0; -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -x_99 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitant_x3f(x_3, x_98, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_99) == 0) -{ -lean_object* x_100; -x_100 = lean_ctor_get(x_99, 0); -lean_inc(x_100); -if (lean_obj_tag(x_100) == 0) -{ -lean_object* x_101; lean_object* x_102; -x_101 = lean_ctor_get(x_99, 1); -lean_inc(x_101); -lean_dec(x_99); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -x_102 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_findAssumption_x3f(x_2, x_3, x_4, x_5, x_6, x_7, x_101); -if (lean_obj_tag(x_102) == 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_104; lean_object* x_105; -x_104 = lean_ctor_get(x_102, 1); -lean_inc(x_104); -lean_dec(x_102); -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_105 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkFnInhabitant_x3f(x_2, x_3, x_98, x_4, x_5, x_6, x_7, x_104); -if (lean_obj_tag(x_105) == 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_107; lean_object* x_108; -x_107 = lean_ctor_get(x_105, 1); -lean_inc(x_107); -lean_dec(x_105); -x_108 = lean_box(0); -x_9 = x_108; -x_10 = x_107; -goto block_97; +if (lean_is_scalar(x_113)) { + x_114 = lean_alloc_ctor(1, 2, 0); +} else { + x_114 = x_113; } -else -{ -lean_object* x_109; uint8_t x_110; -x_109 = lean_ctor_get(x_105, 1); -lean_inc(x_109); -lean_dec(x_105); -x_110 = !lean_is_exclusive(x_106); -if (x_110 == 0) -{ -x_9 = x_106; -x_10 = x_109; -goto block_97; +lean_ctor_set(x_114, 0, x_111); +lean_ctor_set(x_114, 1, x_112); +return x_114; } -else -{ -lean_object* x_111; lean_object* x_112; -x_111 = lean_ctor_get(x_106, 0); -lean_inc(x_111); -lean_dec(x_106); -x_112 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_112, 0, x_111); -x_9 = x_112; -x_10 = x_109; -goto block_97; } } } else { -uint8_t x_113; +uint8_t x_115; lean_dec(x_7); +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_113 = !lean_is_exclusive(x_105); -if (x_113 == 0) +x_115 = !lean_is_exclusive(x_40); +if (x_115 == 0) { -return x_105; +return x_40; } else { -lean_object* x_114; lean_object* x_115; lean_object* x_116; -x_114 = lean_ctor_get(x_105, 0); -x_115 = lean_ctor_get(x_105, 1); -lean_inc(x_115); -lean_inc(x_114); -lean_dec(x_105); -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_116; lean_object* x_117; lean_object* x_118; +x_116 = lean_ctor_get(x_40, 0); +x_117 = lean_ctor_get(x_40, 1); +lean_inc(x_117); +lean_inc(x_116); +lean_dec(x_40); +x_118 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_118, 0, x_116); +lean_ctor_set(x_118, 1, x_117); +return x_118; } } } else { -lean_object* x_117; uint8_t x_118; -x_117 = lean_ctor_get(x_102, 1); -lean_inc(x_117); -lean_dec(x_102); -x_118 = !lean_is_exclusive(x_103); -if (x_118 == 0) -{ -lean_object* x_119; uint8_t x_120; uint8_t x_121; lean_object* x_122; -x_119 = lean_ctor_get(x_103, 0); -x_120 = 1; -x_121 = 1; -lean_inc(x_2); -x_122 = l_Lean_Meta_mkLambdaFVars(x_2, x_119, x_98, x_120, x_98, x_121, x_4, x_5, x_6, x_7, x_117); +lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; +lean_dec(x_7); +x_119 = lean_unsigned_to_nat(1u); +x_120 = lean_nat_add(x_13, x_119); +lean_dec(x_13); +x_121 = lean_alloc_ctor(0, 12, 2); +lean_ctor_set(x_121, 0, x_10); +lean_ctor_set(x_121, 1, x_11); +lean_ctor_set(x_121, 2, x_12); +lean_ctor_set(x_121, 3, x_120); +lean_ctor_set(x_121, 4, x_14); +lean_ctor_set(x_121, 5, x_15); +lean_ctor_set(x_121, 6, x_16); +lean_ctor_set(x_121, 7, x_17); +lean_ctor_set(x_121, 8, x_18); +lean_ctor_set(x_121, 9, x_19); +lean_ctor_set(x_121, 10, x_20); +lean_ctor_set(x_121, 11, x_22); +lean_ctor_set_uint8(x_121, sizeof(void*)*12, x_21); +lean_ctor_set_uint8(x_121, sizeof(void*)*12 + 1, x_23); +lean_inc(x_8); +lean_inc(x_121); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_3); +x_122 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitant_x3f(x_3, x_4, x_5, x_6, x_121, x_8, x_9); if (lean_obj_tag(x_122) == 0) { -lean_object* x_123; lean_object* x_124; +lean_object* x_123; x_123 = lean_ctor_get(x_122, 0); lean_inc(x_123); +if (lean_obj_tag(x_123) == 0) +{ +lean_object* x_124; lean_object* x_125; lean_object* x_126; x_124 = lean_ctor_get(x_122, 1); lean_inc(x_124); lean_dec(x_122); -lean_ctor_set(x_103, 0, x_123); -x_9 = x_103; -x_10 = x_124; -goto block_97; -} -else +x_125 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___closed__1; +lean_inc(x_8); +lean_inc(x_121); +lean_inc(x_6); +lean_inc(x_5); +x_126 = l_Lean_Meta_whnfEasyCases___at_Lean_Meta_whnfCore_go___spec__2(x_125, x_3, x_125, x_5, x_6, x_121, x_8, x_124); +if (lean_obj_tag(x_126) == 0) { -uint8_t x_125; -lean_free_object(x_103); -lean_dec(x_7); +lean_object* x_127; lean_object* x_128; uint8_t x_129; +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_Expr_isForall(x_127); +if (x_129 == 0) +{ +lean_object* x_130; +lean_inc(x_8); +lean_inc(x_121); +lean_inc(x_6); +lean_inc(x_5); +x_130 = l_Lean_Meta_unfoldDefinition_x3f(x_127, x_5, x_6, x_121, x_8, x_128); +if (lean_obj_tag(x_130) == 0) +{ +lean_object* x_131; +x_131 = lean_ctor_get(x_130, 0); +lean_inc(x_131); +if (lean_obj_tag(x_131) == 0) +{ +lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; +lean_dec(x_121); +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_125 = !lean_is_exclusive(x_122); -if (x_125 == 0) -{ -return x_122; -} -else -{ -lean_object* x_126; lean_object* x_127; lean_object* x_128; -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_alloc_ctor(1, 2, 0); -lean_ctor_set(x_128, 0, x_126); -lean_ctor_set(x_128, 1, x_127); -return x_128; +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_box(0); +if (lean_is_scalar(x_133)) { + x_135 = lean_alloc_ctor(0, 2, 0); +} else { + x_135 = x_133; } +lean_ctor_set(x_135, 0, x_134); +lean_ctor_set(x_135, 1, x_132); +return x_135; } else { -lean_object* x_129; uint8_t x_130; uint8_t x_131; lean_object* x_132; -x_129 = lean_ctor_get(x_103, 0); -lean_inc(x_129); -lean_dec(x_103); -x_130 = 1; -x_131 = 1; -lean_inc(x_2); -x_132 = l_Lean_Meta_mkLambdaFVars(x_2, x_129, x_98, x_130, x_98, x_131, x_4, x_5, x_6, x_7, x_117); -if (lean_obj_tag(x_132) == 0) -{ -lean_object* x_133; lean_object* x_134; lean_object* x_135; -x_133 = lean_ctor_get(x_132, 0); -lean_inc(x_133); -x_134 = lean_ctor_get(x_132, 1); -lean_inc(x_134); -lean_dec(x_132); -x_135 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_135, 0, x_133); -x_9 = x_135; -x_10 = x_134; -goto block_97; +lean_object* x_136; lean_object* x_137; +x_136 = lean_ctor_get(x_130, 1); +lean_inc(x_136); +lean_dec(x_130); +x_137 = lean_ctor_get(x_131, 0); +lean_inc(x_137); +lean_dec(x_131); +x_3 = x_137; +x_7 = x_121; +x_9 = x_136; +goto _start; +} } else { -lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; -lean_dec(x_7); +lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; +lean_dec(x_121); +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_136 = lean_ctor_get(x_132, 0); -lean_inc(x_136); -x_137 = lean_ctor_get(x_132, 1); -lean_inc(x_137); -if (lean_is_exclusive(x_132)) { - lean_ctor_release(x_132, 0); - lean_ctor_release(x_132, 1); - x_138 = x_132; +x_139 = lean_ctor_get(x_130, 0); +lean_inc(x_139); +x_140 = lean_ctor_get(x_130, 1); +lean_inc(x_140); +if (lean_is_exclusive(x_130)) { + lean_ctor_release(x_130, 0); + lean_ctor_release(x_130, 1); + x_141 = x_130; } else { - lean_dec_ref(x_132); - x_138 = lean_box(0); + lean_dec_ref(x_130); + x_141 = lean_box(0); } -if (lean_is_scalar(x_138)) { - x_139 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_141)) { + x_142 = lean_alloc_ctor(1, 2, 0); } else { - x_139 = x_138; + x_142 = x_141; } -lean_ctor_set(x_139, 0, x_136); -lean_ctor_set(x_139, 1, x_137); -return x_139; +lean_ctor_set(x_142, 0, x_139); +lean_ctor_set(x_142, 1, x_140); +return x_142; } } +else +{ +lean_object* x_143; lean_object* x_144; uint8_t x_145; lean_object* x_146; +x_143 = lean_box(x_4); +x_144 = lean_alloc_closure((void*)(l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___lambda__2___boxed), 10, 3); +lean_closure_set(x_144, 0, x_1); +lean_closure_set(x_144, 1, x_2); +lean_closure_set(x_144, 2, x_143); +x_145 = 0; +x_146 = l_Lean_Meta_forallTelescope___at_Lean_Meta_mapForallTelescope_x27___spec__1___rarg(x_127, x_144, x_145, x_5, x_6, x_121, x_8, x_128); +return x_146; } } else { -uint8_t x_140; -lean_dec(x_7); +lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; +lean_dec(x_121); +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_140 = !lean_is_exclusive(x_102); -if (x_140 == 0) -{ -return x_102; +x_147 = lean_ctor_get(x_126, 0); +lean_inc(x_147); +x_148 = lean_ctor_get(x_126, 1); +lean_inc(x_148); +if (lean_is_exclusive(x_126)) { + lean_ctor_release(x_126, 0); + lean_ctor_release(x_126, 1); + x_149 = x_126; +} else { + lean_dec_ref(x_126); + x_149 = lean_box(0); } -else -{ -lean_object* x_141; lean_object* x_142; lean_object* x_143; -x_141 = lean_ctor_get(x_102, 0); -x_142 = lean_ctor_get(x_102, 1); -lean_inc(x_142); -lean_inc(x_141); -lean_dec(x_102); -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; +if (lean_is_scalar(x_149)) { + x_150 = lean_alloc_ctor(1, 2, 0); +} else { + x_150 = x_149; } +lean_ctor_set(x_150, 0, x_147); +lean_ctor_set(x_150, 1, x_148); +return x_150; } } else { -lean_object* x_144; uint8_t x_145; -x_144 = lean_ctor_get(x_99, 1); -lean_inc(x_144); -lean_dec(x_99); -x_145 = !lean_is_exclusive(x_100); -if (x_145 == 0) -{ -lean_object* x_146; uint8_t x_147; uint8_t x_148; lean_object* x_149; -x_146 = lean_ctor_get(x_100, 0); -x_147 = 1; -x_148 = 1; -lean_inc(x_2); -x_149 = l_Lean_Meta_mkLambdaFVars(x_2, x_146, x_98, x_147, x_98, x_148, x_4, x_5, x_6, x_7, x_144); -if (lean_obj_tag(x_149) == 0) -{ -lean_object* x_150; lean_object* x_151; -x_150 = lean_ctor_get(x_149, 0); -lean_inc(x_150); -x_151 = lean_ctor_get(x_149, 1); +lean_object* x_151; lean_object* x_152; lean_object* x_153; uint8_t x_154; uint8_t x_155; uint8_t x_156; lean_object* x_157; +lean_dec(x_3); +x_151 = lean_ctor_get(x_122, 1); lean_inc(x_151); -lean_dec(x_149); -lean_ctor_set(x_100, 0, x_150); -x_9 = x_100; -x_10 = x_151; -goto block_97; -} -else -{ -uint8_t x_152; -lean_free_object(x_100); -lean_dec(x_7); +lean_dec(x_122); +x_152 = lean_ctor_get(x_123, 0); +lean_inc(x_152); +if (lean_is_exclusive(x_123)) { + lean_ctor_release(x_123, 0); + x_153 = x_123; +} else { + lean_dec_ref(x_123); + x_153 = lean_box(0); +} +x_154 = 0; +x_155 = 1; +x_156 = 1; +x_157 = l_Lean_Meta_mkLambdaFVars(x_2, x_152, x_154, x_155, x_154, x_156, x_5, x_6, x_121, x_8, x_151); +if (lean_obj_tag(x_157) == 0) +{ +lean_object* x_158; lean_object* x_159; lean_object* x_160; +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_Meta_mkLambdaFVars(x_1, x_158, x_154, x_155, x_154, x_156, x_5, x_6, x_121, x_8, x_159); +lean_dec(x_8); +lean_dec(x_121); 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_152 = !lean_is_exclusive(x_149); -if (x_152 == 0) +if (lean_obj_tag(x_160) == 0) { -return x_149; +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_160, 0); +lean_inc(x_161); +x_162 = lean_ctor_get(x_160, 1); +lean_inc(x_162); +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); } -else -{ -lean_object* x_153; lean_object* x_154; lean_object* x_155; -x_153 = lean_ctor_get(x_149, 0); -x_154 = lean_ctor_get(x_149, 1); -lean_inc(x_154); -lean_inc(x_153); -lean_dec(x_149); -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; +if (lean_is_scalar(x_153)) { + x_164 = lean_alloc_ctor(1, 1, 0); +} else { + x_164 = x_153; } +lean_ctor_set(x_164, 0, x_161); +if (lean_is_scalar(x_163)) { + x_165 = lean_alloc_ctor(0, 2, 0); +} else { + x_165 = x_163; } +lean_ctor_set(x_165, 0, x_164); +lean_ctor_set(x_165, 1, x_162); +return x_165; } else { -lean_object* x_156; uint8_t x_157; uint8_t x_158; lean_object* x_159; -x_156 = lean_ctor_get(x_100, 0); -lean_inc(x_156); -lean_dec(x_100); -x_157 = 1; -x_158 = 1; -lean_inc(x_2); -x_159 = l_Lean_Meta_mkLambdaFVars(x_2, x_156, x_98, x_157, x_98, x_158, x_4, x_5, x_6, x_7, x_144); -if (lean_obj_tag(x_159) == 0) -{ -lean_object* x_160; lean_object* x_161; lean_object* x_162; -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_alloc_ctor(1, 1, 0); -lean_ctor_set(x_162, 0, x_160); -x_9 = x_162; -x_10 = x_161; -goto block_97; +lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; +lean_dec(x_153); +x_166 = lean_ctor_get(x_160, 0); +lean_inc(x_166); +x_167 = lean_ctor_get(x_160, 1); +lean_inc(x_167); +if (lean_is_exclusive(x_160)) { + lean_ctor_release(x_160, 0); + lean_ctor_release(x_160, 1); + x_168 = x_160; +} else { + lean_dec_ref(x_160); + x_168 = lean_box(0); +} +if (lean_is_scalar(x_168)) { + x_169 = lean_alloc_ctor(1, 2, 0); +} else { + x_169 = x_168; +} +lean_ctor_set(x_169, 0, x_166); +lean_ctor_set(x_169, 1, x_167); +return x_169; +} } else { -lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; -lean_dec(x_7); +lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; +lean_dec(x_153); +lean_dec(x_121); +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_163 = lean_ctor_get(x_159, 0); -lean_inc(x_163); -x_164 = lean_ctor_get(x_159, 1); -lean_inc(x_164); -if (lean_is_exclusive(x_159)) { - lean_ctor_release(x_159, 0); - lean_ctor_release(x_159, 1); - x_165 = x_159; +x_170 = lean_ctor_get(x_157, 0); +lean_inc(x_170); +x_171 = lean_ctor_get(x_157, 1); +lean_inc(x_171); +if (lean_is_exclusive(x_157)) { + lean_ctor_release(x_157, 0); + lean_ctor_release(x_157, 1); + x_172 = x_157; } else { - lean_dec_ref(x_159); - x_165 = lean_box(0); + lean_dec_ref(x_157); + x_172 = lean_box(0); } -if (lean_is_scalar(x_165)) { - x_166 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_172)) { + x_173 = lean_alloc_ctor(1, 2, 0); } else { - x_166 = x_165; -} -lean_ctor_set(x_166, 0, x_163); -lean_ctor_set(x_166, 1, x_164); -return x_166; + x_173 = x_172; } +lean_ctor_set(x_173, 0, x_170); +lean_ctor_set(x_173, 1, x_171); +return x_173; } } } else { -uint8_t x_167; -lean_dec(x_7); +lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; +lean_dec(x_121); +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_167 = !lean_is_exclusive(x_99); -if (x_167 == 0) -{ -return x_99; +x_174 = lean_ctor_get(x_122, 0); +lean_inc(x_174); +x_175 = lean_ctor_get(x_122, 1); +lean_inc(x_175); +if (lean_is_exclusive(x_122)) { + lean_ctor_release(x_122, 0); + lean_ctor_release(x_122, 1); + x_176 = x_122; +} else { + lean_dec_ref(x_122); + x_176 = lean_box(0); } -else -{ -lean_object* x_168; lean_object* x_169; lean_object* x_170; -x_168 = lean_ctor_get(x_99, 0); -x_169 = lean_ctor_get(x_99, 1); -lean_inc(x_169); -lean_inc(x_168); -lean_dec(x_99); -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; +if (lean_is_scalar(x_176)) { + x_177 = lean_alloc_ctor(1, 2, 0); +} else { + x_177 = x_176; } +lean_ctor_set(x_177, 0, x_174); +lean_ctor_set(x_177, 1, x_175); +return x_177; } -block_97: -{ -if (lean_obj_tag(x_9) == 0) -{ -lean_object* x_11; lean_object* x_12; uint8_t x_22; lean_object* x_23; -x_22 = 1; -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -x_23 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitant_x3f(x_3, x_22, x_4, x_5, x_6, x_7, x_10); -if (lean_obj_tag(x_23) == 0) -{ -lean_object* x_24; -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -if (lean_obj_tag(x_24) == 0) -{ -lean_object* x_25; lean_object* x_26; -x_25 = lean_ctor_get(x_23, 1); -lean_inc(x_25); -lean_dec(x_23); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -x_26 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_findAssumption_x3f(x_2, x_3, x_4, x_5, x_6, x_7, x_25); -if (lean_obj_tag(x_26) == 0) -{ -lean_object* x_27; -x_27 = lean_ctor_get(x_26, 0); -lean_inc(x_27); -if (lean_obj_tag(x_27) == 0) -{ -lean_object* x_28; lean_object* x_29; -x_28 = lean_ctor_get(x_26, 1); -lean_inc(x_28); -lean_dec(x_26); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -x_29 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkFnInhabitant_x3f(x_2, x_3, x_22, x_4, x_5, x_6, x_7, x_28); -if (lean_obj_tag(x_29) == 0) -{ -lean_object* x_30; -x_30 = lean_ctor_get(x_29, 0); -lean_inc(x_30); -if (lean_obj_tag(x_30) == 0) -{ -lean_object* x_31; lean_object* x_32; -x_31 = lean_ctor_get(x_29, 1); -lean_inc(x_31); -lean_dec(x_29); -x_32 = lean_box(0); -x_11 = x_32; -x_12 = x_31; -goto block_21; } -else -{ -lean_object* x_33; uint8_t x_34; -x_33 = lean_ctor_get(x_29, 1); -lean_inc(x_33); -lean_dec(x_29); -x_34 = !lean_is_exclusive(x_30); -if (x_34 == 0) -{ -x_11 = x_30; -x_12 = x_33; -goto block_21; } else { -lean_object* x_35; lean_object* x_36; -x_35 = lean_ctor_get(x_30, 0); -lean_inc(x_35); -lean_dec(x_30); -x_36 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_36, 0, x_35); -x_11 = x_36; -x_12 = x_33; -goto block_21; +lean_object* x_178; +lean_dec(x_22); +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_178 = l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1(x_15, 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); +return x_178; } } } -else +LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___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: { -uint8_t x_37; -lean_dec(x_7); -lean_dec(x_6); +lean_object* x_7; +x_7 = l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_1); -x_37 = !lean_is_exclusive(x_29); -if (x_37 == 0) -{ -return x_29; +lean_dec(x_3); +lean_dec(x_2); +return x_7; } -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_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +uint8_t x_12; lean_object* x_13; +x_12 = lean_unbox(x_5); +lean_dec(x_5); +x_13 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___lambda__1(x_1, x_2, x_3, x_4, x_12, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_6); +lean_dec(x_2); +return x_13; } } -else +LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: { -lean_object* x_41; uint8_t x_42; +uint8_t x_11; lean_object* x_12; +x_11 = lean_unbox(x_3); lean_dec(x_3); -x_41 = lean_ctor_get(x_26, 1); -lean_inc(x_41); -lean_dec(x_26); -x_42 = !lean_is_exclusive(x_27); -if (x_42 == 0) -{ -lean_object* x_43; uint8_t x_44; uint8_t x_45; lean_object* x_46; -x_43 = lean_ctor_get(x_27, 0); -x_44 = 0; -x_45 = 1; -x_46 = l_Lean_Meta_mkLambdaFVars(x_2, x_43, x_44, x_22, x_44, x_45, x_4, x_5, x_6, x_7, x_41); -if (lean_obj_tag(x_46) == 0) -{ -lean_object* x_47; lean_object* x_48; -x_47 = lean_ctor_get(x_46, 0); -lean_inc(x_47); -x_48 = lean_ctor_get(x_46, 1); -lean_inc(x_48); -lean_dec(x_46); -lean_ctor_set(x_27, 0, x_47); -x_11 = x_27; -x_12 = x_48; -goto block_21; +x_12 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___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; } -else +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: { -uint8_t x_49; -lean_free_object(x_27); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); +uint8_t x_10; lean_object* x_11; +x_10 = lean_unbox(x_4); lean_dec(x_4); -lean_dec(x_1); -x_49 = !lean_is_exclusive(x_46); -if (x_49 == 0) -{ -return x_46; +x_11 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f(x_1, x_2, x_3, x_10, x_5, x_6, x_7, x_8, x_9); +return x_11; } -else +} +static lean_object* _init_l_Lean_Elab_mkInhabitantFor___lambda__1___closed__1() { +_start: { -lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_50 = lean_ctor_get(x_46, 0); -x_51 = lean_ctor_get(x_46, 1); -lean_inc(x_51); -lean_inc(x_50); -lean_dec(x_46); -x_52 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_52, 0, x_50); -lean_ctor_set(x_52, 1, x_51); -return x_52; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("failed to compile 'partial' definition '", 40, 40); +return x_1; } } +static lean_object* _init_l_Lean_Elab_mkInhabitantFor___lambda__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_mkInhabitantFor___lambda__1___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} } -else +static lean_object* _init_l_Lean_Elab_mkInhabitantFor___lambda__1___closed__3() { +_start: { -lean_object* x_53; uint8_t x_54; uint8_t x_55; lean_object* x_56; -x_53 = lean_ctor_get(x_27, 0); -lean_inc(x_53); -lean_dec(x_27); -x_54 = 0; -x_55 = 1; -x_56 = l_Lean_Meta_mkLambdaFVars(x_2, x_53, x_54, x_22, x_54, x_55, x_4, x_5, x_6, x_7, x_41); -if (lean_obj_tag(x_56) == 0) +lean_object* x_1; +x_1 = lean_mk_string_unchecked("', could not prove that the type", 32, 32); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_mkInhabitantFor___lambda__1___closed__4() { +_start: { -lean_object* x_57; lean_object* x_58; lean_object* x_59; -x_57 = lean_ctor_get(x_56, 0); -lean_inc(x_57); -x_58 = lean_ctor_get(x_56, 1); -lean_inc(x_58); -lean_dec(x_56); -x_59 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_59, 0, x_57); -x_11 = x_59; -x_12 = x_58; -goto block_21; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_mkInhabitantFor___lambda__1___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } -else +} +static lean_object* _init_l_Lean_Elab_mkInhabitantFor___lambda__1___closed__5() { +_start: { -lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_1); -x_60 = lean_ctor_get(x_56, 0); -lean_inc(x_60); -x_61 = lean_ctor_get(x_56, 1); -lean_inc(x_61); -if (lean_is_exclusive(x_56)) { - lean_ctor_release(x_56, 0); - lean_ctor_release(x_56, 1); - x_62 = x_56; -} else { - lean_dec_ref(x_56); - x_62 = lean_box(0); +lean_object* x_1; +x_1 = lean_mk_string_unchecked("\nis nonempty.\n\nThis process uses multiple strategies:\n- It looks for a parameter that matches the return type.\n- It tries synthesizing '", 136, 136); +return x_1; } -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; +static lean_object* _init_l_Lean_Elab_mkInhabitantFor___lambda__1___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_mkInhabitantFor___lambda__1___closed__5; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } +static lean_object* _init_l_Lean_Elab_mkInhabitantFor___lambda__1___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__2; +x_2 = l_Lean_MessageData_ofConstName(x_1); +return x_2; } } -else +static lean_object* _init_l_Lean_Elab_mkInhabitantFor___lambda__1___closed__8() { +_start: { -uint8_t x_64; -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_64 = !lean_is_exclusive(x_26); -if (x_64 == 0) +lean_object* x_1; +x_1 = lean_mk_string_unchecked("' and '", 7, 7); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_mkInhabitantFor___lambda__1___closed__9() { +_start: { -return x_26; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_mkInhabitantFor___lambda__1___closed__8; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } -else +} +static lean_object* _init_l_Lean_Elab_mkInhabitantFor___lambda__1___closed__10() { +_start: { -lean_object* x_65; lean_object* x_66; lean_object* x_67; -x_65 = lean_ctor_get(x_26, 0); -x_66 = lean_ctor_get(x_26, 1); -lean_inc(x_66); -lean_inc(x_65); -lean_dec(x_26); -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_1; +x_1 = lean_mk_string_unchecked("Nonempty", 8, 8); +return x_1; } } +static lean_object* _init_l_Lean_Elab_mkInhabitantFor___lambda__1___closed__11() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_mkInhabitantFor___lambda__1___closed__10; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} } -else +static lean_object* _init_l_Lean_Elab_mkInhabitantFor___lambda__1___closed__12() { +_start: { -lean_object* x_68; uint8_t x_69; -lean_dec(x_3); -x_68 = lean_ctor_get(x_23, 1); -lean_inc(x_68); -lean_dec(x_23); -x_69 = !lean_is_exclusive(x_24); -if (x_69 == 0) -{ -lean_object* x_70; uint8_t x_71; uint8_t x_72; lean_object* x_73; -x_70 = lean_ctor_get(x_24, 0); -x_71 = 0; -x_72 = 1; -x_73 = l_Lean_Meta_mkLambdaFVars(x_2, x_70, x_71, x_22, x_71, x_72, x_4, x_5, x_6, x_7, x_68); -if (lean_obj_tag(x_73) == 0) -{ -lean_object* x_74; lean_object* x_75; -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_ctor_set(x_24, 0, x_74); -x_11 = x_24; -x_12 = x_75; -goto block_21; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_mkInhabitantFor___lambda__1___closed__11; +x_2 = l_Lean_MessageData_ofConstName(x_1); +return x_2; } -else +} +static lean_object* _init_l_Lean_Elab_mkInhabitantFor___lambda__1___closed__13() { +_start: { -uint8_t x_76; -lean_free_object(x_24); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_1); -x_76 = !lean_is_exclusive(x_73); -if (x_76 == 0) +lean_object* x_1; +x_1 = lean_mk_string_unchecked("' instances for the return type, while making every parameter into a local '", 76, 76); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_mkInhabitantFor___lambda__1___closed__14() { +_start: { -return x_73; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_mkInhabitantFor___lambda__1___closed__13; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } -else +} +static lean_object* _init_l_Lean_Elab_mkInhabitantFor___lambda__1___closed__15() { +_start: { -lean_object* x_77; lean_object* x_78; lean_object* x_79; -x_77 = lean_ctor_get(x_73, 0); -x_78 = lean_ctor_get(x_73, 1); -lean_inc(x_78); -lean_inc(x_77); -lean_dec(x_73); -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_1; +x_1 = lean_mk_string_unchecked("' instance.\n- It tries unfolding the return type.\n\nIf the return type is defined using the 'structure' or 'inductive' command, you can try adding a 'deriving Nonempty' clause to it.", 181, 181); +return x_1; } } +static lean_object* _init_l_Lean_Elab_mkInhabitantFor___lambda__1___closed__16() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_mkInhabitantFor___lambda__1___closed__15; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } -else +} +LEAN_EXPORT lean_object* l_Lean_Elab_mkInhabitantFor___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_80; uint8_t x_81; uint8_t x_82; lean_object* x_83; -x_80 = lean_ctor_get(x_24, 0); -lean_inc(x_80); -lean_dec(x_24); -x_81 = 0; -x_82 = 1; -x_83 = l_Lean_Meta_mkLambdaFVars(x_2, x_80, x_81, x_22, x_81, x_82, x_4, x_5, x_6, x_7, x_68); -if (lean_obj_tag(x_83) == 0) -{ -lean_object* x_84; lean_object* x_85; lean_object* x_86; -x_84 = lean_ctor_get(x_83, 0); -lean_inc(x_84); -x_85 = lean_ctor_get(x_83, 1); -lean_inc(x_85); -lean_dec(x_83); -x_86 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_86, 0, x_84); -x_11 = x_86; -x_12 = x_85; -goto block_21; +lean_object* x_10; lean_object* x_11; uint8_t x_46; lean_object* x_47; +x_46 = 0; +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_2); +lean_inc(x_4); +lean_inc(x_1); +x_47 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f(x_1, x_4, x_2, x_46, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_47) == 0) +{ +lean_object* x_48; +x_48 = lean_ctor_get(x_47, 0); +lean_inc(x_48); +if (lean_obj_tag(x_48) == 0) +{ +lean_object* x_49; uint8_t x_50; lean_object* x_51; +x_49 = lean_ctor_get(x_47, 1); +lean_inc(x_49); +lean_dec(x_47); +x_50 = 1; +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_2); +lean_inc(x_1); +x_51 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f(x_1, x_4, x_2, x_50, x_5, x_6, x_7, x_8, x_49); +if (lean_obj_tag(x_51) == 0) +{ +lean_object* x_52; lean_object* x_53; +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_10 = x_52; +x_11 = x_53; +goto block_45; } else { -lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; +uint8_t x_54; +lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); lean_dec(x_1); -x_87 = lean_ctor_get(x_83, 0); -lean_inc(x_87); -x_88 = lean_ctor_get(x_83, 1); -lean_inc(x_88); -if (lean_is_exclusive(x_83)) { - lean_ctor_release(x_83, 0); - lean_ctor_release(x_83, 1); - x_89 = x_83; -} else { - lean_dec_ref(x_83); - x_89 = lean_box(0); +x_54 = !lean_is_exclusive(x_51); +if (x_54 == 0) +{ +return x_51; } -if (lean_is_scalar(x_89)) { - x_90 = lean_alloc_ctor(1, 2, 0); -} else { - x_90 = x_89; +else +{ +lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_55 = lean_ctor_get(x_51, 0); +x_56 = lean_ctor_get(x_51, 1); +lean_inc(x_56); +lean_inc(x_55); +lean_dec(x_51); +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_ctor_set(x_90, 0, x_87); -lean_ctor_set(x_90, 1, x_88); -return x_90; } } +else +{ +lean_object* x_58; +lean_dec(x_4); +x_58 = lean_ctor_get(x_47, 1); +lean_inc(x_58); +lean_dec(x_47); +x_10 = x_48; +x_11 = x_58; +goto block_45; } } else { -uint8_t x_91; +uint8_t x_59; +lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -1894,86 +1785,153 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_91 = !lean_is_exclusive(x_23); -if (x_91 == 0) +x_59 = !lean_is_exclusive(x_47); +if (x_59 == 0) { -return x_23; +return x_47; } else { -lean_object* x_92; lean_object* x_93; lean_object* x_94; -x_92 = lean_ctor_get(x_23, 0); -x_93 = lean_ctor_get(x_23, 1); -lean_inc(x_93); -lean_inc(x_92); -lean_dec(x_23); -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; +lean_object* x_60; lean_object* x_61; lean_object* x_62; +x_60 = lean_ctor_get(x_47, 0); +x_61 = lean_ctor_get(x_47, 1); +lean_inc(x_61); +lean_inc(x_60); +lean_dec(x_47); +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; } } -block_21: +block_45: { -if (lean_obj_tag(x_11) == 0) +if (lean_obj_tag(x_10) == 0) +{ +uint8_t x_12; uint8_t x_13; uint8_t x_14; lean_object* x_15; +x_12 = 0; +x_13 = 1; +x_14 = 1; +x_15 = l_Lean_Meta_mkForallFVars(x_1, x_2, x_12, x_13, x_14, x_5, x_6, x_7, x_8, x_11); +if (lean_obj_tag(x_15) == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_13 = l_Lean_MessageData_ofName(x_1); -x_14 = l_Lean_Elab_mkInhabitantFor___closed__2; -x_15 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_15, 0, x_14); -lean_ctor_set(x_15, 1, x_13); -x_16 = l_Lean_Elab_mkInhabitantFor___closed__4; -x_17 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_17, 0, x_15); -lean_ctor_set(x_17, 1, x_16); -x_18 = l_Lean_throwError___at_Lean_Expr_abstractRangeM___spec__1(x_17, x_4, x_5, x_6, x_7, x_12); +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_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_MessageData_ofName(x_3); +x_19 = l_Lean_Elab_mkInhabitantFor___lambda__1___closed__2; +x_20 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_20, 0, x_19); +lean_ctor_set(x_20, 1, x_18); +x_21 = l_Lean_Elab_mkInhabitantFor___lambda__1___closed__4; +x_22 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_22, 0, x_20); +lean_ctor_set(x_22, 1, x_21); +x_23 = l_Lean_indentExpr(x_16); +x_24 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); +x_25 = l_Lean_Elab_mkInhabitantFor___lambda__1___closed__6; +x_26 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_26, 0, x_24); +lean_ctor_set(x_26, 1, x_25); +x_27 = l_Lean_Elab_mkInhabitantFor___lambda__1___closed__7; +x_28 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +x_29 = l_Lean_Elab_mkInhabitantFor___lambda__1___closed__9; +x_30 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +x_31 = l_Lean_Elab_mkInhabitantFor___lambda__1___closed__12; +x_32 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_31); +x_33 = l_Lean_Elab_mkInhabitantFor___lambda__1___closed__14; +x_34 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_34, 0, x_32); +lean_ctor_set(x_34, 1, x_33); +x_35 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_35, 0, x_34); +lean_ctor_set(x_35, 1, x_27); +x_36 = l_Lean_Elab_mkInhabitantFor___lambda__1___closed__16; +x_37 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +x_38 = l_Lean_throwError___at_Lean_Expr_abstractRangeM___spec__1(x_37, x_5, x_6, x_7, x_8, x_17); +lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); -return x_18; +return x_38; } else { -lean_object* x_19; lean_object* x_20; +uint8_t x_39; +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_19 = lean_ctor_get(x_11, 0); -lean_inc(x_19); -lean_dec(x_11); -x_20 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_20, 0, x_19); -lean_ctor_set(x_20, 1, x_12); -return x_20; +lean_dec(x_3); +x_39 = !lean_is_exclusive(x_15); +if (x_39 == 0) +{ +return x_15; +} +else +{ +lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_40 = lean_ctor_get(x_15, 0); +x_41 = lean_ctor_get(x_15, 1); +lean_inc(x_41); +lean_inc(x_40); +lean_dec(x_15); +x_42 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_42, 0, x_40); +lean_ctor_set(x_42, 1, x_41); +return x_42; } } } else { -lean_object* x_95; lean_object* x_96; +lean_object* x_43; lean_object* x_44; +lean_dec(x_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_95 = lean_ctor_get(x_9, 0); -lean_inc(x_95); -lean_dec(x_9); -x_96 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_96, 0, x_95); -lean_ctor_set(x_96, 1, x_10); -return x_96; +x_43 = lean_ctor_get(x_10, 0); +lean_inc(x_43); +lean_dec(x_10); +x_44 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_44, 0, x_43); +lean_ctor_set(x_44, 1, x_11); +return x_44; +} +} } } +LEAN_EXPORT lean_object* l_Lean_Elab_mkInhabitantFor(lean_object* x_1, lean_object* x_2, lean_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_inc(x_2); +x_9 = lean_alloc_closure((void*)(l_Lean_Elab_mkInhabitantFor___lambda__1), 9, 3); +lean_closure_set(x_9, 0, x_2); +lean_closure_set(x_9, 1, x_3); +lean_closure_set(x_9, 2, x_1); +x_10 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances___rarg(x_2, x_9, x_4, x_5, x_6, x_7, x_8); +return x_10; } } lean_object* initialize_Lean_Meta_AppBuilder(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_PrettyPrinter(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Lean_Elab_PreDefinition_MkInhabitant(uint8_t builtin, lean_object* w) { lean_object * res; @@ -1982,16 +1940,69 @@ _G_initialized = true; res = initialize_Lean_Meta_AppBuilder(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_findAssumption_x3f___closed__1 = _init_l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_findAssumption_x3f___closed__1(); -lean_mark_persistent(l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_findAssumption_x3f___closed__1); -l_Lean_Elab_mkInhabitantFor___closed__1 = _init_l_Lean_Elab_mkInhabitantFor___closed__1(); -lean_mark_persistent(l_Lean_Elab_mkInhabitantFor___closed__1); -l_Lean_Elab_mkInhabitantFor___closed__2 = _init_l_Lean_Elab_mkInhabitantFor___closed__2(); -lean_mark_persistent(l_Lean_Elab_mkInhabitantFor___closed__2); -l_Lean_Elab_mkInhabitantFor___closed__3 = _init_l_Lean_Elab_mkInhabitantFor___closed__3(); -lean_mark_persistent(l_Lean_Elab_mkInhabitantFor___closed__3); -l_Lean_Elab_mkInhabitantFor___closed__4 = _init_l_Lean_Elab_mkInhabitantFor___closed__4(); -lean_mark_persistent(l_Lean_Elab_mkInhabitantFor___closed__4); +res = initialize_Lean_PrettyPrinter(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__1 = _init_l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__1(); +lean_mark_persistent(l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__1); +l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__2 = _init_l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__2(); +lean_mark_persistent(l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__2); +l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__3 = _init_l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__3(); +lean_mark_persistent(l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__3); +l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__4 = _init_l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__4(); +lean_mark_persistent(l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__4); +l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__5 = _init_l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__5(); +lean_mark_persistent(l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__5); +l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__6 = _init_l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__6(); +lean_mark_persistent(l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances_go___rarg___closed__6); +l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances___rarg___closed__1 = _init_l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances___rarg___closed__1(); +lean_mark_persistent(l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_withInhabitedInstances___rarg___closed__1); +l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__1 = _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__1(); +lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__1); +l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__2 = _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__2(); +lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__2); +l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__3 = _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__3(); +lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__3); +l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__4 = _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__4(); +lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__4); +l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__5 = _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__5(); +lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__5); +l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__6 = _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__6(); +lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___spec__1___closed__6); +l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___closed__1 = _init_l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___closed__1(); +lean_mark_persistent(l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkInhabitantForAux_x3f___closed__1); +l_Lean_Elab_mkInhabitantFor___lambda__1___closed__1 = _init_l_Lean_Elab_mkInhabitantFor___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Elab_mkInhabitantFor___lambda__1___closed__1); +l_Lean_Elab_mkInhabitantFor___lambda__1___closed__2 = _init_l_Lean_Elab_mkInhabitantFor___lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Elab_mkInhabitantFor___lambda__1___closed__2); +l_Lean_Elab_mkInhabitantFor___lambda__1___closed__3 = _init_l_Lean_Elab_mkInhabitantFor___lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Elab_mkInhabitantFor___lambda__1___closed__3); +l_Lean_Elab_mkInhabitantFor___lambda__1___closed__4 = _init_l_Lean_Elab_mkInhabitantFor___lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Elab_mkInhabitantFor___lambda__1___closed__4); +l_Lean_Elab_mkInhabitantFor___lambda__1___closed__5 = _init_l_Lean_Elab_mkInhabitantFor___lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Elab_mkInhabitantFor___lambda__1___closed__5); +l_Lean_Elab_mkInhabitantFor___lambda__1___closed__6 = _init_l_Lean_Elab_mkInhabitantFor___lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Elab_mkInhabitantFor___lambda__1___closed__6); +l_Lean_Elab_mkInhabitantFor___lambda__1___closed__7 = _init_l_Lean_Elab_mkInhabitantFor___lambda__1___closed__7(); +lean_mark_persistent(l_Lean_Elab_mkInhabitantFor___lambda__1___closed__7); +l_Lean_Elab_mkInhabitantFor___lambda__1___closed__8 = _init_l_Lean_Elab_mkInhabitantFor___lambda__1___closed__8(); +lean_mark_persistent(l_Lean_Elab_mkInhabitantFor___lambda__1___closed__8); +l_Lean_Elab_mkInhabitantFor___lambda__1___closed__9 = _init_l_Lean_Elab_mkInhabitantFor___lambda__1___closed__9(); +lean_mark_persistent(l_Lean_Elab_mkInhabitantFor___lambda__1___closed__9); +l_Lean_Elab_mkInhabitantFor___lambda__1___closed__10 = _init_l_Lean_Elab_mkInhabitantFor___lambda__1___closed__10(); +lean_mark_persistent(l_Lean_Elab_mkInhabitantFor___lambda__1___closed__10); +l_Lean_Elab_mkInhabitantFor___lambda__1___closed__11 = _init_l_Lean_Elab_mkInhabitantFor___lambda__1___closed__11(); +lean_mark_persistent(l_Lean_Elab_mkInhabitantFor___lambda__1___closed__11); +l_Lean_Elab_mkInhabitantFor___lambda__1___closed__12 = _init_l_Lean_Elab_mkInhabitantFor___lambda__1___closed__12(); +lean_mark_persistent(l_Lean_Elab_mkInhabitantFor___lambda__1___closed__12); +l_Lean_Elab_mkInhabitantFor___lambda__1___closed__13 = _init_l_Lean_Elab_mkInhabitantFor___lambda__1___closed__13(); +lean_mark_persistent(l_Lean_Elab_mkInhabitantFor___lambda__1___closed__13); +l_Lean_Elab_mkInhabitantFor___lambda__1___closed__14 = _init_l_Lean_Elab_mkInhabitantFor___lambda__1___closed__14(); +lean_mark_persistent(l_Lean_Elab_mkInhabitantFor___lambda__1___closed__14); +l_Lean_Elab_mkInhabitantFor___lambda__1___closed__15 = _init_l_Lean_Elab_mkInhabitantFor___lambda__1___closed__15(); +lean_mark_persistent(l_Lean_Elab_mkInhabitantFor___lambda__1___closed__15); +l_Lean_Elab_mkInhabitantFor___lambda__1___closed__16 = _init_l_Lean_Elab_mkInhabitantFor___lambda__1___closed__16(); +lean_mark_persistent(l_Lean_Elab_mkInhabitantFor___lambda__1___closed__16); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/Structural/BRecOn.c b/stage0/stdlib/Lean/Elab/PreDefinition/Structural/BRecOn.c index 57cfbf73de8f..30aa1081783f 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/Structural/BRecOn.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/Structural/BRecOn.c @@ -19,6 +19,7 @@ lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__10___boxed(lean_object*); lean_object* l_Lean_Meta_inferArgumentTypesN(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Structural_mkBrecOnApp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__4(lean_object*); @@ -38,6 +39,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_getMatcherInfo_x3f___at___private_Lean_Elab static lean_object* l_Lean_Elab_Structural_mkBrecOnApp___lambda__2___closed__5; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Structural_mkBRecOnConst___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Structural_mkBRecOnConst___lambda__5(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__27(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___lambda__5___closed__4; lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); @@ -54,6 +56,7 @@ lean_object* l_Lean_Elab_Structural_IndGroupInfo_numMotives(lean_object*); uint8_t l_Lean_Exception_isInterrupt(lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___closed__7; static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__39___lambda__3___closed__1; +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_isExprDefEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_lambdaBoundedTelescope___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__38___rarg(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -62,6 +65,7 @@ lean_object* l_Lean_Elab_Structural_RecArgInfo_pickIndicesMajor(lean_object*, le static lean_object* l_Lean_getConstInfo___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__3___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Structural_inferBRecOnFTypes___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Structural_mkBRecOnConst___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_forallBoundedTelescope___at_Lean_Elab_Structural_mkBRecOnF___spec__1___rarg(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_findIdx_x3f_loop___rarg(lean_object*, lean_object*, lean_object*); @@ -80,7 +84,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Structural_Positions_mapMwith___at___privat static lean_object* l_panic___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__5___closed__1; static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___lambda__5___closed__3; uint8_t lean_usize_dec_eq(size_t, size_t); -static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__2; lean_object* l_Lean_Expr_mdata___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__13(lean_object*); static lean_object* l_Lean_Elab_Structural_searchPProd___rarg___closed__4; @@ -88,8 +91,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Structural_inferBRecOnFTypes___lambda__1(le lean_object* l_Lean_replaceRef(lean_object*, lean_object*); uint8_t l_Array_contains___at_Lean_Elab_Structural_RecArgInfo_pickIndicesMajor___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__12(lean_object*); -static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___closed__2; -static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__5; +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_isTracingEnabledFor___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__35___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_addTrace___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__40___boxed(lean_object*); lean_object* l_Lean_Expr_proj___override(lean_object*, lean_object*, lean_object*); @@ -103,8 +105,10 @@ extern lean_object* l_Lean_casesOnSuffix; lean_object* l_Lean_Meta_Match_MatcherInfo_arity(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__25___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__3(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__4; LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__13___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__4___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_environment_find(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_getMatcherInfo_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -126,6 +130,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0 LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__43(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_addTrace___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__40___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__22___lambda__1(lean_object*, lean_object*); +static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__5; lean_object* l_Nat_nextPowerOfTwo_go(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps___spec__1(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -137,18 +142,15 @@ LEAN_EXPORT lean_object* l_Lean_addTrace___at___private_Lean_Elab_PreDefinition_ lean_object* l_Lean_stringToMessageData(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__31___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12(lean_object*); LEAN_EXPORT uint8_t l_Array_getIdx_x3f___at_Lean_Elab_Structural_mkBrecOnApp___spec__6___lambda__1(lean_object*, lean_object*); uint8_t l___private_Lean_Util_Trace_0__Lean_checkTraceOption(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_getConstInfoInduct___at_Lean_Elab_Structural_mkBRecOnConst___spec__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__11___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__7___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__7___closed__2; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__9(size_t, size_t, lean_object*); uint8_t lean_string_dec_eq(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___lambda__5___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -157,7 +159,6 @@ LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_PreDefinition_Structur LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__26___boxed(lean_object*); extern lean_object* l_Lean_Elab_Structural_instInhabitedRecArgInfo; static lean_object* l_Lean_Elab_Structural_Positions_mapMwith___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__4___closed__7; -static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Structural_mkBRecOnF___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static double l_Lean_addTrace___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__37___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__31___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -167,14 +168,13 @@ static lean_object* l_List_forIn_loop___at___private_Lean_Elab_PreDefinition_Str LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Structural_searchPProd___rarg___closed__2; extern lean_object* l_instInhabitedPUnit; -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__14___closed__1; +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__36___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_lambdaTelescope___at_Lean_Elab_Structural_mkBRecOnMotive___spec__1___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Structural_IndGroupInst_brecOn(lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_throwToBelowFailed___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Structural_Positions_mapMwith___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__4___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelow___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_isTypeCorrect(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -191,20 +191,18 @@ static lean_object* l_Lean_Elab_Structural_mkBrecOnApp___lambda__2___closed__9; lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_lambdaTelescopeImp___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_panic___at_String_toNat_x21___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__21___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10(lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__22(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__41(lean_object*, lean_object*); +static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4___closed__2; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__33___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Structural_mkBRecOnF___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__39___lambda__2___closed__4; lean_object* l_Lean_throwError___at_Lean_Expr_abstractRangeM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_take(lean_object*, lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withLetDeclImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__41___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5___closed__1; -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_expr_eqv(lean_object*, lean_object*); @@ -218,7 +216,7 @@ static lean_object* l_Lean_Elab_Structural_Positions_mapMwith___at___private_Lea static lean_object* l_Lean_Elab_Structural_searchPProd___rarg___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__39(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__41___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4___closed__1; +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8(lean_object*); lean_object* l_Lean_Meta_PProdN_proj(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -226,6 +224,7 @@ static lean_object* l_Lean_Elab_Structural_mkBrecOnApp___lambda__2___closed__7; LEAN_EXPORT lean_object* l_Lean_isTracingEnabledFor___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__29___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Structural_mkBRecOnConst___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_throwToBelowFailed___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_getIdx_x3f___at_Lean_Elab_Structural_mkBrecOnApp___spec__6___lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__7(lean_object*); @@ -235,10 +234,12 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefi LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__28___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_SavedState_restore(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withLocalDeclImp___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_getPrefix(lean_object*); LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__13___boxed(lean_object*); lean_object* l___private_Lean_CoreM_0__Lean_Core_mkFreshNameImp(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_isTracingEnabledFor___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__35___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___closed__2; lean_object* l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__23(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -258,6 +259,7 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Structural_mkBr LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__1(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__22___lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__17(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_throwToBelowFailed___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__18___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -286,7 +288,9 @@ static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lea extern lean_object* l_Lean_instInhabitedExpr; LEAN_EXPORT lean_object* l_Lean_Elab_Structural_inferBRecOnFTypes(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Structural_mkBRecOnConst___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__43___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_lengthTRAux___rarg(lean_object*, lean_object*); @@ -301,7 +305,6 @@ lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__22___closed__2; lean_object* l_Lean_Meta_lambdaTelescope___at_Lean_PrettyPrinter_Delaborator_returnsPi___spec__1___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__24(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__41___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Structural_inferBRecOnFTypes___closed__2; LEAN_EXPORT lean_object* l_Lean_addTrace___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__40___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -309,10 +312,12 @@ static lean_object* l_Lean_Elab_Structural_Positions_mapMwith___at___private_Lea static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__9___closed__1; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__19(lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__5___closed__2; +static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5___closed__2; lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__5___closed__1; static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__3___closed__1; lean_object* l_Lean_Meta_PProdN_packLambdas(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps___spec__1___boxed(lean_object*, lean_object*, lean_object*); @@ -325,24 +330,19 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinitio LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__42___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Structural_mkBrecOnApp___lambda__2___closed__1; extern lean_object* l_Lean_Meta_instMonadMetaM; -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__2; static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__19___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2___closed__1; LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__8(lean_object*); static lean_object* l_Lean_Elab_Structural_searchPProd___rarg___closed__5; LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__22___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Structural_mkBrecOnApp___lambda__1___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Meta_forallTelescopeCompatibleAux___spec__15___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__1; LEAN_EXPORT lean_object* l_Lean_addTrace___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__37___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___closed__6; -static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4___closed__2; static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__39___lambda__3___closed__4; lean_object* l_Array_append___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__11___boxed(lean_object*); -static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__3; extern lean_object* l_Lean_inheritedTraceOptions; static lean_object* l_Lean_Elab_Structural_mkBrecOnApp___lambda__2___closed__8; lean_object* l_Lean_MessageData_ofExpr(lean_object*); @@ -352,9 +352,9 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefi LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__20___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__7___closed__3; LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_Structural_mkBrecOnApp___spec__4(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); double l_Float_ofScientific(lean_object*, uint8_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__26(lean_object*); -static lean_object* l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg___closed__1; lean_object* l_Array_extract___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__39___lambda__2___closed__1; LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__9___boxed(lean_object*); @@ -365,17 +365,16 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Structural_mkBRecOnMotive___lambda__1(lean_ static lean_object* l_Lean_Elab_Structural_mkBrecOnApp___lambda__2___closed__2; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__33___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__21___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_addTrace___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__37___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__39___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__14___closed__2; lean_object* l_Lean_Expr_replaceFVars(lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__3___closed__2; -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__34___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelow(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_zetaReduce___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Structural_inferBRecOnFTypes___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__4___closed__2; @@ -391,7 +390,6 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinitio LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__6(lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_lambdaTelescope___at_Lean_Elab_Structural_mkBRecOnMotive___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__11(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Structural_inferBRecOnFTypes___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_getConstInfo___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__3___closed__1; LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -419,12 +417,11 @@ static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lea lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__42(lean_object*, lean_object*); lean_object* l_Lean_Meta_MatcherApp_toExpr(lean_object*); +static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__32(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_zetaReduce___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_lambdaBoundedTelescope___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__38___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_panic_fn(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__11___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__3(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -435,6 +432,7 @@ static lean_object* l_Lean_Elab_Structural_mkBrecOnApp___lambda__2___closed__6; LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__27___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_panic___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__7___rarg___closed__3; +static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2___closed__2; static lean_object* l_Lean_Elab_Structural_Positions_mapMwith___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__4___closed__8; LEAN_EXPORT lean_object* l_Lean_getConstInfoInduct___at_Lean_Elab_Structural_mkBRecOnConst___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_addTrace___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__37(lean_object*); @@ -454,23 +452,18 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0 LEAN_EXPORT lean_object* l_Lean_Elab_Structural_searchPProd___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_mk(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___lambda__1___boxed(lean_object**); -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5___closed__2; LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__8___boxed(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); -static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__4; static lean_object* l_panic___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__7___rarg___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__26___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_ensureNoRecFn(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_throwToBelowFailed___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_instInhabitedName; -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_uget(lean_object*, size_t); size_t lean_array_size(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__9___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__4___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_throwToBelowFailed___rarg___closed__1; @@ -486,8 +479,8 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Structural_searchPProd(lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallTelescopeReducingAux___rarg(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_lambdaTelescope___at_Lean_Elab_Structural_mkBRecOnMotive___spec__1(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__7___boxed(lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Structural_mkBRecOnConst___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -513,7 +506,6 @@ lean_object* l_Lean_Meta_mkLambdaFVars(lean_object*, lean_object*, uint8_t, uint LEAN_EXPORT lean_object* l_Lean_Meta_getMatcherInfo_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__16(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_getIdx_x3f___at_Lean_Elab_Structural_mkBrecOnApp___spec__6___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___closed__3; @@ -521,14 +513,13 @@ uint8_t l_Lean_Exception_isRuntime(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Structural_inferBRecOnFTypes___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__18(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__39___lambda__3___boxed(lean_object**); static lean_object* l_Lean_Elab_Structural_mkBrecOnApp___lambda__2___closed__11; -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_panic___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__7___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__19___boxed(lean_object*); lean_object* l_Lean_InductiveVal_numCtors(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_lambdaBoundedTelescope___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__38___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__3; static lean_object* l_Lean_Elab_Structural_mkBRecOnF___lambda__2___closed__1; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___closed__5; @@ -539,7 +530,7 @@ lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_instantiateForallAux(lean_ LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__43___rarg(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Structural_Positions_mapMwith___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__4___closed__9; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__39___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__2; lean_object* l_ReaderT_instMonad___rarg(lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__4___closed__4; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__33___boxed(lean_object*); @@ -2805,218 +2796,7 @@ return x_24; } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__9(size_t x_1, size_t x_2, lean_object* x_3) { -_start: -{ -uint8_t x_4; -x_4 = lean_usize_dec_lt(x_2, x_1); -if (x_4 == 0) -{ -return x_3; -} -else -{ -lean_object* x_5; lean_object* x_6; lean_object* x_7; size_t x_8; size_t x_9; uint8_t x_10; -x_5 = lean_array_uget(x_3, x_2); -x_6 = lean_unsigned_to_nat(0u); -x_7 = lean_array_uset(x_3, x_2, x_6); -x_8 = 1; -x_9 = lean_usize_add(x_2, x_8); -x_10 = !lean_is_exclusive(x_5); -if (x_10 == 0) -{ -lean_object* x_11; uint8_t x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_11 = lean_ctor_get(x_5, 0); -x_12 = 0; -x_13 = lean_box(x_12); -lean_ctor_set(x_5, 0, x_13); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_11); -lean_ctor_set(x_14, 1, x_5); -x_15 = lean_array_uset(x_7, x_2, x_14); -x_2 = x_9; -x_3 = x_15; -goto _start; -} -else -{ -lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_17 = lean_ctor_get(x_5, 0); -x_18 = lean_ctor_get(x_5, 1); -lean_inc(x_18); -lean_inc(x_17); -lean_dec(x_5); -x_19 = 0; -x_20 = lean_box(x_19); -x_21 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_21, 0, x_20); -lean_ctor_set(x_21, 1, x_18); -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_17); -lean_ctor_set(x_22, 1, x_21); -x_23 = lean_array_uset(x_7, x_2, x_22); -x_2 = x_9; -x_3 = x_23; -goto _start; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__11___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; lean_object* x_12; -x_11 = lean_array_push(x_1, x_5); -x_12 = l_Lean_Meta_withLocalDecls_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__11___rarg(x_2, x_3, x_4, x_11, x_6, x_7, x_8, x_9, x_10); -return x_12; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__11___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_10 = lean_array_get_size(x_4); -x_11 = lean_array_get_size(x_1); -x_12 = lean_nat_dec_lt(x_10, x_11); -lean_dec(x_11); -if (x_12 == 0) -{ -lean_object* x_13; -lean_dec(x_10); -lean_dec(x_3); -lean_dec(x_1); -x_13 = lean_apply_6(x_2, x_4, x_5, x_6, x_7, x_8, x_9); -return x_13; -} -else -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_14 = lean_array_fget(x_1, x_10); -lean_dec(x_10); -x_15 = lean_ctor_get(x_14, 1); -lean_inc(x_15); -x_16 = lean_ctor_get(x_14, 0); -lean_inc(x_16); -lean_dec(x_14); -x_17 = lean_ctor_get(x_15, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_15, 1); -lean_inc(x_18); -lean_dec(x_15); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -x_19 = lean_apply_6(x_18, x_4, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_19) == 0) -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; uint8_t x_24; lean_object* x_25; -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_19, 1); -lean_inc(x_21); -lean_dec(x_19); -x_22 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecls_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__11___rarg___lambda__1), 10, 4); -lean_closure_set(x_22, 0, x_4); -lean_closure_set(x_22, 1, x_1); -lean_closure_set(x_22, 2, x_2); -lean_closure_set(x_22, 3, x_3); -x_23 = 0; -x_24 = lean_unbox(x_17); -lean_dec(x_17); -x_25 = l_Lean_Meta_withLocalDecl___at_Lean_Meta_forallTelescopeCompatibleAux___spec__15___rarg(x_16, x_24, x_20, x_22, x_23, x_5, x_6, x_7, x_8, x_21); -return x_25; -} -else -{ -uint8_t x_26; -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_26 = !lean_is_exclusive(x_19); -if (x_26 == 0) -{ -return x_19; -} -else -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_19, 0); -x_28 = lean_ctor_get(x_19, 1); -lean_inc(x_28); -lean_inc(x_27); -lean_dec(x_19); -x_29 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_29, 0, x_27); -lean_ctor_set(x_29, 1, x_28); -return x_29; -} -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__11(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecls_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__11___rarg), 9, 0); -return x_2; -} -} -static lean_object* _init_l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = lean_box(0); -x_2 = lean_array_mk(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; lean_object* x_10; -x_9 = l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg___closed__1; -x_10 = l_Lean_Meta_withLocalDecls_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__11___rarg(x_2, x_3, x_1, x_9, x_4, x_5, x_6, x_7, x_8); -return x_10; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg), 8, 0); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -size_t x_9; size_t x_10; lean_object* x_11; lean_object* x_12; -x_9 = lean_array_size(x_2); -x_10 = 0; -x_11 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__9(x_9, x_10, x_2); -x_12 = l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg(x_1, x_11, x_3, x_4, x_5, x_6, x_7, x_8); -return x_12; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDeclsD___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg), 8, 0); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { lean_object* x_10; @@ -3024,7 +2804,7 @@ x_10 = lean_apply_7(x_1, x_2, x_3, x_5, x_6, x_7, x_8, x_9); return x_10; } } -static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2___closed__1() { +static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2___closed__1() { _start: { lean_object* x_1; @@ -3032,16 +2812,16 @@ x_1 = lean_mk_string_unchecked("not type correct!", 17, 17); return x_1; } } -static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2___closed__2() { +static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2___closed__1; +x_1 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; @@ -3086,7 +2866,7 @@ lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean x_20 = lean_ctor_get(x_15, 1); lean_inc(x_20); lean_dec(x_15); -x_21 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2___closed__2; +x_21 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2___closed__2; x_22 = l_Lean_addTrace___at_Lean_Meta_processPostponed_loop___spec__2(x_4, x_21, x_6, x_7, x_8, x_9, x_20); x_23 = lean_ctor_get(x_22, 1); lean_inc(x_23); @@ -3138,7 +2918,7 @@ return x_30; } } } -static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__1() { +static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__1() { _start: { lean_object* x_1; @@ -3146,7 +2926,7 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Meta_PProdN_packLambdas), 7, 0); return x_1; } } -static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__2() { +static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__2() { _start: { lean_object* x_1; @@ -3154,16 +2934,16 @@ x_1 = lean_mk_string_unchecked("initial belowDict for ", 22, 22); return x_1; } } -static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__3() { +static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__2; +x_1 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__2; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__4() { +static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__4() { _start: { lean_object* x_1; @@ -3171,21 +2951,21 @@ x_1 = lean_mk_string_unchecked(":", 1, 1); return x_1; } } -static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__5() { +static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__5() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__4; +x_1 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__4; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; lean_object* x_15; x_13 = l_Lean_instInhabitedExpr; -x_14 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__1; +x_14 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__1; lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); @@ -3217,7 +2997,7 @@ x_24 = lean_ctor_get(x_21, 1); lean_inc(x_24); lean_dec(x_21); x_25 = lean_box(0); -x_26 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2(x_20, x_6, x_7, x_5, x_25, x_8, x_9, x_10, x_11, x_24); +x_26 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2(x_20, x_6, x_7, x_5, x_25, x_8, x_9, x_10, x_11, x_24); return x_26; } else @@ -3235,11 +3015,11 @@ x_30 = lean_array_to_list(x_7); x_31 = lean_box(0); x_32 = l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(x_30, x_31); x_33 = l_Lean_MessageData_ofList(x_32); -x_34 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__3; +x_34 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__3; lean_ctor_set_tag(x_21, 7); lean_ctor_set(x_21, 1, x_33); lean_ctor_set(x_21, 0, x_34); -x_35 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__5; +x_35 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__5; x_36 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_36, 0, x_21); lean_ctor_set(x_36, 1, x_35); @@ -3259,7 +3039,7 @@ lean_inc(x_42); x_43 = lean_ctor_get(x_41, 1); lean_inc(x_43); lean_dec(x_41); -x_44 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2(x_20, x_6, x_7, x_5, x_42, x_8, x_9, x_10, x_11, x_43); +x_44 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2(x_20, x_6, x_7, x_5, x_42, x_8, x_9, x_10, x_11, x_43); lean_dec(x_42); return x_44; } @@ -3274,11 +3054,11 @@ x_46 = lean_array_to_list(x_7); x_47 = lean_box(0); x_48 = l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(x_46, x_47); x_49 = l_Lean_MessageData_ofList(x_48); -x_50 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__3; +x_50 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__3; x_51 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_51, 0, x_50); lean_ctor_set(x_51, 1, x_49); -x_52 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__5; +x_52 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__5; x_53 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_53, 0, x_51); lean_ctor_set(x_53, 1, x_52); @@ -3298,7 +3078,7 @@ lean_inc(x_59); x_60 = lean_ctor_get(x_58, 1); lean_inc(x_60); lean_dec(x_58); -x_61 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2(x_20, x_6, x_7, x_5, x_59, x_8, x_9, x_10, x_11, x_60); +x_61 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2(x_20, x_6, x_7, x_5, x_59, x_8, x_9, x_10, x_11, x_60); lean_dec(x_59); return x_61; } @@ -3336,7 +3116,7 @@ return x_65; } } } -static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4___closed__1() { +static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4___closed__1() { _start: { lean_object* x_1; lean_object* x_2; @@ -3345,20 +3125,20 @@ x_2 = l_Lean_Level_ofNat(x_1); return x_2; } } -static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4___closed__2() { +static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4___closed__1; +x_1 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4___closed__1; x_2 = l_Lean_Expr_sort___override(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; size_t x_21; size_t x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; size_t x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_15 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4___closed__2; +x_15 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4___closed__2; x_16 = lean_mk_array(x_1, x_15); x_17 = lean_array_get_size(x_2); x_18 = lean_unsigned_to_nat(0u); @@ -3385,18 +3165,18 @@ lean_inc(x_29); x_30 = lean_ctor_get(x_28, 1); lean_inc(x_30); lean_dec(x_28); -x_31 = lean_alloc_closure((void*)(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___boxed), 12, 6); +x_31 = lean_alloc_closure((void*)(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___boxed), 12, 6); lean_closure_set(x_31, 0, x_3); lean_closure_set(x_31, 1, x_2); lean_closure_set(x_31, 2, x_4); lean_closure_set(x_31, 3, x_5); lean_closure_set(x_31, 4, x_6); lean_closure_set(x_31, 5, x_7); -x_32 = l_Lean_Meta_withLocalDeclsD___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg(x_8, x_29, x_31, x_10, x_11, x_12, x_13, x_30); +x_32 = l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__2___rarg(x_8, x_29, x_31, x_10, x_11, x_12, x_13, x_30); return x_32; } } -static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5___closed__1() { +static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5___closed__1() { _start: { lean_object* x_1; @@ -3404,16 +3184,16 @@ x_1 = lean_mk_string_unchecked("numMotives: ", 12, 12); return x_1; } } -static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5___closed__2() { +static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5___closed__1; +x_1 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; @@ -3457,7 +3237,7 @@ x_29 = lean_ctor_get(x_26, 1); lean_inc(x_29); lean_dec(x_26); x_30 = lean_box(0); -x_31 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4(x_25, x_23, x_5, x_21, x_19, x_6, x_7, x_8, x_30, x_10, x_11, x_12, x_13, x_29); +x_31 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4(x_25, x_23, x_5, x_21, x_19, x_6, x_7, x_8, x_30, x_10, x_11, x_12, x_13, x_29); return x_31; } else @@ -3475,7 +3255,7 @@ x_35 = l___private_Init_Data_Repr_0__Nat_reprFast(x_25); x_36 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_36, 0, x_35); x_37 = l_Lean_MessageData_ofFormat(x_36); -x_38 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5___closed__2; +x_38 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5___closed__2; lean_ctor_set_tag(x_26, 7); lean_ctor_set(x_26, 1, x_37); lean_ctor_set(x_26, 0, x_38); @@ -3490,7 +3270,7 @@ lean_inc(x_42); x_43 = lean_ctor_get(x_41, 1); lean_inc(x_43); lean_dec(x_41); -x_44 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4(x_25, x_23, x_5, x_21, x_19, x_6, x_7, x_8, x_42, x_10, x_11, x_12, x_13, x_43); +x_44 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4(x_25, x_23, x_5, x_21, x_19, x_6, x_7, x_8, x_42, x_10, x_11, x_12, x_13, x_43); lean_dec(x_42); return x_44; } @@ -3505,7 +3285,7 @@ x_46 = l___private_Init_Data_Repr_0__Nat_reprFast(x_25); x_47 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_47, 0, x_46); x_48 = l_Lean_MessageData_ofFormat(x_47); -x_49 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5___closed__2; +x_49 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5___closed__2; x_50 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_50, 0, x_49); lean_ctor_set(x_50, 1, x_48); @@ -3520,7 +3300,7 @@ lean_inc(x_54); x_55 = lean_ctor_get(x_53, 1); lean_inc(x_55); lean_dec(x_53); -x_56 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4(x_25, x_23, x_5, x_21, x_19, x_6, x_7, x_8, x_54, x_10, x_11, x_12, x_13, x_55); +x_56 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4(x_25, x_23, x_5, x_21, x_19, x_6, x_7, x_8, x_54, x_10, x_11, x_12, x_13, x_55); lean_dec(x_54); return x_56; } @@ -3560,7 +3340,7 @@ return x_60; } } } -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; uint8_t x_9; @@ -3585,7 +3365,7 @@ return x_12; } } } -static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___closed__1() { +static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___closed__1() { _start: { lean_object* x_1; @@ -3593,16 +3373,16 @@ x_1 = lean_mk_string_unchecked("unexpected 'below' type", 23, 23); return x_1; } } -static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___closed__2() { +static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___closed__1; +x_1 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { if (lean_obj_tag(x_8) == 5) @@ -3634,7 +3414,7 @@ lean_inc(x_8); lean_inc(x_5); lean_inc(x_2); lean_inc(x_9); -x_22 = lean_alloc_closure((void*)(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5___boxed), 14, 8); +x_22 = lean_alloc_closure((void*)(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5___boxed), 14, 8); lean_closure_set(x_22, 0, x_9); lean_closure_set(x_22, 1, x_2); lean_closure_set(x_22, 2, x_5); @@ -3673,7 +3453,7 @@ x_29 = lean_ctor_get(x_26, 1); lean_inc(x_29); lean_dec(x_26); x_30 = lean_box(0); -x_31 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__6(x_22, x_30, x_11, x_12, x_13, x_14, x_29); +x_31 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__6(x_22, x_30, x_11, x_12, x_13, x_14, x_29); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); @@ -3692,7 +3472,7 @@ x_33 = lean_ctor_get(x_26, 1); x_34 = lean_ctor_get(x_26, 0); lean_dec(x_34); x_35 = l_Lean_indentExpr(x_6); -x_36 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___closed__2; +x_36 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___closed__2; lean_ctor_set_tag(x_26, 7); lean_ctor_set(x_26, 1, x_35); lean_ctor_set(x_26, 0, x_36); @@ -3706,7 +3486,7 @@ lean_inc(x_40); x_41 = lean_ctor_get(x_39, 1); lean_inc(x_41); lean_dec(x_39); -x_42 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__6(x_22, x_40, x_11, x_12, x_13, x_14, x_41); +x_42 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__6(x_22, x_40, x_11, x_12, x_13, x_14, x_41); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); @@ -3722,7 +3502,7 @@ x_43 = lean_ctor_get(x_26, 1); lean_inc(x_43); lean_dec(x_26); x_44 = l_Lean_indentExpr(x_6); -x_45 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___closed__2; +x_45 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___closed__2; x_46 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_46, 0, x_45); lean_ctor_set(x_46, 1, x_44); @@ -3736,7 +3516,7 @@ lean_inc(x_50); x_51 = lean_ctor_get(x_49, 1); lean_inc(x_51); lean_dec(x_49); -x_52 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__6(x_22, x_50, x_11, x_12, x_13, x_14, x_51); +x_52 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__6(x_22, x_50, x_11, x_12, x_13, x_14, x_51); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); @@ -3753,17 +3533,17 @@ lean_object* x_53; lean_object* x_54; lean_dec(x_22); lean_dec(x_6); x_53 = lean_box(0); -x_54 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5(x_9, x_2, x_5, x_8, x_3, x_7, x_4, x_1, x_53, x_11, x_12, x_13, x_14, x_15); +x_54 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5(x_9, x_2, x_5, x_8, x_3, x_7, x_4, x_1, x_53, x_11, x_12, x_13, x_14, x_15); return x_54; } } } } -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg), 15, 0); +x_2 = lean_alloc_closure((void*)(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg), 15, 0); return x_2; } } @@ -3780,7 +3560,7 @@ x_18 = lean_unsigned_to_nat(1u); x_19 = lean_nat_sub(x_15, x_18); lean_dec(x_15); lean_inc(x_1); -x_20 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg(x_2, x_3, x_4, x_5, x_6, x_1, x_7, x_1, x_17, x_19, x_9, x_10, x_11, x_12, x_13); +x_20 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg(x_2, x_3, x_4, x_5, x_6, x_1, x_7, x_1, x_17, x_19, x_9, x_10, x_11, x_12, x_13); return x_20; } } @@ -3828,7 +3608,7 @@ lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean x_25 = lean_ctor_get(x_19, 1); lean_inc(x_25); lean_dec(x_19); -x_26 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2___closed__2; +x_26 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2___closed__2; lean_inc(x_8); x_27 = l_Lean_addTrace___at_Lean_Meta_processPostponed_loop___spec__2(x_8, x_26, x_10, x_11, x_12, x_13, x_25); x_28 = lean_ctor_get(x_27, 0); @@ -4128,70 +3908,58 @@ lean_dec(x_3); return x_11; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -size_t x_4; size_t x_5; lean_object* x_6; -x_4 = lean_unbox_usize(x_1); -lean_dec(x_1); -x_5 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__9(x_4, x_5, x_3); -return x_6; -} -} -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { lean_object* x_10; -x_10 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_10 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_4); return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; -x_11 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_5); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; -x_13 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_13 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); return x_13; } } -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { lean_object* x_15; -x_15 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +x_15 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); lean_dec(x_9); return x_15; } } -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { lean_object* x_15; -x_15 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +x_15 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); lean_dec(x_9); return x_15; } } -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; -x_8 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); @@ -8785,6 +8553,15 @@ static lean_object* _init_l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_El _start: { lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_array_mk(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; x_1 = lean_unsigned_to_nat(0u); x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); @@ -8851,7 +8628,7 @@ x_40 = l_outOfBounds___rarg(x_39); if (x_37 == 0) { lean_object* x_41; lean_object* x_42; -x_41 = l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg___closed__1; +x_41 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__1; x_42 = l_List_forIn_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__14(x_4, x_38, x_41, x_7, x_8, x_9, x_10, x_11, x_12, x_13); if (lean_obj_tag(x_42) == 0) { @@ -8870,7 +8647,7 @@ x_48 = l_Array_ofSubarray___rarg(x_30); lean_dec(x_30); x_49 = l_Array_ofSubarray___rarg(x_32); lean_dec(x_32); -x_50 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__1; +x_50 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__2; x_51 = lean_alloc_ctor(0, 10, 0); lean_ctor_set(x_51, 0, x_5); lean_ctor_set(x_51, 1, x_45); @@ -8904,7 +8681,7 @@ x_58 = l_Array_ofSubarray___rarg(x_30); lean_dec(x_30); x_59 = l_Array_ofSubarray___rarg(x_32); lean_dec(x_32); -x_60 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__1; +x_60 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__2; x_61 = lean_alloc_ctor(0, 10, 0); lean_ctor_set(x_61, 0, x_5); lean_ctor_set(x_61, 1, x_55); @@ -8958,7 +8735,7 @@ return x_67; else { lean_object* x_68; lean_object* x_69; -x_68 = l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg___closed__1; +x_68 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__1; x_69 = l_List_forIn_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__15(x_4, x_38, x_68, x_7, x_8, x_9, x_10, x_11, x_12, x_13); if (lean_obj_tag(x_69) == 0) { @@ -9073,7 +8850,7 @@ lean_dec(x_2); if (x_37 == 0) { lean_object* x_95; lean_object* x_96; -x_95 = l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg___closed__1; +x_95 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__1; x_96 = l_List_forIn_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__16(x_4, x_93, x_95, x_7, x_8, x_9, x_10, x_11, x_12, x_13); if (lean_obj_tag(x_96) == 0) { @@ -9092,7 +8869,7 @@ x_102 = l_Array_ofSubarray___rarg(x_30); lean_dec(x_30); x_103 = l_Array_ofSubarray___rarg(x_32); lean_dec(x_32); -x_104 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__1; +x_104 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__2; x_105 = lean_alloc_ctor(0, 10, 0); lean_ctor_set(x_105, 0, x_5); lean_ctor_set(x_105, 1, x_99); @@ -9126,7 +8903,7 @@ x_112 = l_Array_ofSubarray___rarg(x_30); lean_dec(x_30); x_113 = l_Array_ofSubarray___rarg(x_32); lean_dec(x_32); -x_114 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__1; +x_114 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__2; x_115 = lean_alloc_ctor(0, 10, 0); lean_ctor_set(x_115, 0, x_5); lean_ctor_set(x_115, 1, x_109); @@ -9180,7 +8957,7 @@ return x_121; else { lean_object* x_122; lean_object* x_123; -x_122 = l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg___closed__1; +x_122 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__1; x_123 = l_List_forIn_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__17(x_4, x_93, x_122, x_7, x_8, x_9, x_10, x_11, x_12, x_13); if (lean_obj_tag(x_123) == 0) { @@ -26022,7 +25799,7 @@ lean_ctor_set(x_23, 1, x_22); lean_ctor_set_float(x_23, sizeof(void*)*2, x_20); lean_ctor_set_float(x_23, sizeof(void*)*2 + 8, x_20); lean_ctor_set_uint8(x_23, sizeof(void*)*2 + 16, x_21); -x_24 = l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg___closed__1; +x_24 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__1; x_25 = lean_alloc_ctor(9, 3, 0); lean_ctor_set(x_25, 0, x_23); lean_ctor_set(x_25, 1, x_12); @@ -26084,7 +25861,7 @@ lean_ctor_set(x_45, 1, x_44); lean_ctor_set_float(x_45, sizeof(void*)*2, x_42); lean_ctor_set_float(x_45, sizeof(void*)*2 + 8, x_42); lean_ctor_set_uint8(x_45, sizeof(void*)*2 + 16, x_43); -x_46 = l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg___closed__1; +x_46 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__1; x_47 = lean_alloc_ctor(9, 3, 0); lean_ctor_set(x_47, 0, x_45); lean_ctor_set(x_47, 1, x_12); @@ -26167,7 +25944,7 @@ lean_ctor_set(x_68, 1, x_67); lean_ctor_set_float(x_68, sizeof(void*)*2, x_65); lean_ctor_set_float(x_68, sizeof(void*)*2 + 8, x_65); lean_ctor_set_uint8(x_68, sizeof(void*)*2 + 16, x_66); -x_69 = l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg___closed__1; +x_69 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__1; x_70 = lean_alloc_ctor(9, 3, 0); lean_ctor_set(x_70, 0, x_68); lean_ctor_set(x_70, 1, x_12); @@ -26817,7 +26594,7 @@ lean_ctor_set(x_23, 1, x_22); lean_ctor_set_float(x_23, sizeof(void*)*2, x_20); lean_ctor_set_float(x_23, sizeof(void*)*2 + 8, x_20); lean_ctor_set_uint8(x_23, sizeof(void*)*2 + 16, x_21); -x_24 = l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg___closed__1; +x_24 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__1; x_25 = lean_alloc_ctor(9, 3, 0); lean_ctor_set(x_25, 0, x_23); lean_ctor_set(x_25, 1, x_12); @@ -26879,7 +26656,7 @@ lean_ctor_set(x_45, 1, x_44); lean_ctor_set_float(x_45, sizeof(void*)*2, x_42); lean_ctor_set_float(x_45, sizeof(void*)*2 + 8, x_42); lean_ctor_set_uint8(x_45, sizeof(void*)*2 + 16, x_43); -x_46 = l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg___closed__1; +x_46 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__1; x_47 = lean_alloc_ctor(9, 3, 0); lean_ctor_set(x_47, 0, x_45); lean_ctor_set(x_47, 1, x_12); @@ -26962,7 +26739,7 @@ lean_ctor_set(x_68, 1, x_67); lean_ctor_set_float(x_68, sizeof(void*)*2, x_65); lean_ctor_set_float(x_68, sizeof(void*)*2 + 8, x_65); lean_ctor_set_uint8(x_68, sizeof(void*)*2 + 16, x_66); -x_69 = l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg___closed__1; +x_69 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__1; x_70 = lean_alloc_ctor(9, 3, 0); lean_ctor_set(x_70, 0, x_68); lean_ctor_set(x_70, 1, x_12); @@ -30414,7 +30191,7 @@ x_17 = lean_ctor_get(x_15, 1); lean_inc(x_17); lean_dec(x_15); x_18 = l_Lean_instInhabitedExpr; -x_19 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__1; +x_19 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__1; x_20 = l_Lean_Elab_Structural_Positions_mapMwith___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__4(x_18, x_19, x_3, x_16, x_4, x_6, x_7, x_8, x_9, x_17); lean_dec(x_16); if (lean_obj_tag(x_20) == 0) @@ -30537,7 +30314,7 @@ x_17 = lean_ctor_get(x_15, 1); lean_inc(x_17); lean_dec(x_15); x_18 = l_Lean_instInhabitedExpr; -x_19 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__1; +x_19 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__1; x_20 = l_Lean_Elab_Structural_Positions_mapMwith___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__4(x_18, x_19, x_4, x_16, x_5, x_7, x_8, x_9, x_10, x_17); lean_dec(x_16); if (lean_obj_tag(x_20) == 0) @@ -31206,248 +30983,216 @@ return x_2; LEAN_EXPORT lean_object* l_Lean_Elab_Structural_inferBRecOnFTypes(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +lean_object* x_9; lean_object* x_10; lean_object* x_57; lean_object* x_58; uint8_t x_59; x_9 = lean_array_get_size(x_2); -x_10 = lean_array_get_size(x_1); -x_11 = lean_unsigned_to_nat(0u); -x_12 = lean_nat_dec_lt(x_11, x_10); -lean_dec(x_10); -x_13 = lean_apply_1(x_3, x_11); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_13); -x_14 = l_Lean_Meta_check(x_13, x_4, x_5, x_6, x_7, x_8); -if (x_12 == 0) -{ -if (lean_obj_tag(x_14) == 0) -{ -lean_object* x_54; lean_object* x_55; lean_object* x_56; -x_54 = lean_ctor_get(x_14, 1); -lean_inc(x_54); -lean_dec(x_14); -x_55 = l_Lean_Elab_Structural_instInhabitedRecArgInfo; -x_56 = l_outOfBounds___rarg(x_55); -x_15 = x_56; -x_16 = x_54; -goto block_53; -} -else -{ -uint8_t x_57; -lean_dec(x_13); -lean_dec(x_9); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); -x_57 = !lean_is_exclusive(x_14); -if (x_57 == 0) +x_57 = lean_array_get_size(x_1); +x_58 = lean_unsigned_to_nat(0u); +x_59 = lean_nat_dec_lt(x_58, x_57); +lean_dec(x_57); +if (x_59 == 0) { -return x_14; +lean_object* x_60; lean_object* x_61; +x_60 = l_Lean_Elab_Structural_instInhabitedRecArgInfo; +x_61 = l_outOfBounds___rarg(x_60); +x_10 = x_61; +goto block_56; } else { -lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_58 = lean_ctor_get(x_14, 0); -x_59 = lean_ctor_get(x_14, 1); -lean_inc(x_59); -lean_inc(x_58); -lean_dec(x_14); -x_60 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_60, 0, x_58); -lean_ctor_set(x_60, 1, x_59); -return x_60; -} -} +lean_object* x_62; +x_62 = lean_array_fget(x_1, x_58); +x_10 = x_62; +goto block_56; } -else -{ -if (lean_obj_tag(x_14) == 0) +block_56: { -lean_object* x_61; lean_object* x_62; -x_61 = lean_ctor_get(x_14, 1); -lean_inc(x_61); -lean_dec(x_14); -x_62 = lean_array_fget(x_1, x_11); -x_15 = x_62; -x_16 = x_61; -goto block_53; -} -else +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_10, 5); +lean_inc(x_11); +x_12 = lean_apply_1(x_3, x_11); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_12); +x_13 = l_Lean_Meta_check(x_12, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_13) == 0) { -uint8_t x_63; +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_13, 1); +lean_inc(x_14); lean_dec(x_13); -lean_dec(x_9); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); -x_63 = !lean_is_exclusive(x_14); -if (x_63 == 0) -{ -return x_14; -} -else -{ -lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_64 = lean_ctor_get(x_14, 0); -x_65 = lean_ctor_get(x_14, 1); -lean_inc(x_65); -lean_inc(x_64); -lean_dec(x_14); -x_66 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_66, 0, x_64); -lean_ctor_set(x_66, 1, x_65); -return x_66; -} -} -} -block_53: -{ -lean_object* x_17; lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -x_17 = lean_infer_type(x_13, x_4, x_5, x_6, x_7, x_16); -if (lean_obj_tag(x_17) == 0) +x_15 = lean_infer_type(x_12, x_4, x_5, x_6, x_7, x_14); +if (lean_obj_tag(x_15) == 0) { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; lean_object* x_27; -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_17, 1); -lean_inc(x_19); -lean_dec(x_17); -x_20 = lean_ctor_get(x_15, 3); -lean_inc(x_20); +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; lean_object* x_25; +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_15, 1); +lean_inc(x_17); lean_dec(x_15); -x_21 = lean_array_get_size(x_20); -lean_dec(x_20); -x_22 = lean_unsigned_to_nat(1u); -x_23 = lean_nat_add(x_21, x_22); -lean_dec(x_21); -x_24 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_24, 0, x_23); +x_18 = lean_ctor_get(x_10, 3); +lean_inc(x_18); +lean_dec(x_10); +x_19 = lean_array_get_size(x_18); +lean_dec(x_18); +x_20 = lean_unsigned_to_nat(1u); +x_21 = lean_nat_add(x_19, x_20); +lean_dec(x_19); +x_22 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_22, 0, x_21); lean_inc(x_9); -x_25 = lean_alloc_closure((void*)(l_Lean_Elab_Structural_inferBRecOnFTypes___lambda__1___boxed), 8, 1); -lean_closure_set(x_25, 0, x_9); -x_26 = 0; +x_23 = lean_alloc_closure((void*)(l_Lean_Elab_Structural_inferBRecOnFTypes___lambda__1___boxed), 8, 1); +lean_closure_set(x_23, 0, x_9); +x_24 = 0; lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -x_27 = l_Lean_Meta_forallBoundedTelescope___at_Lean_Meta_arrowDomainsN___spec__6___rarg(x_18, x_24, x_25, x_26, x_4, x_5, x_6, x_7, x_19); -if (lean_obj_tag(x_27) == 0) +x_25 = l_Lean_Meta_forallBoundedTelescope___at_Lean_Meta_arrowDomainsN___spec__6___rarg(x_16, x_22, x_23, x_24, x_4, x_5, x_6, x_7, x_17); +if (lean_obj_tag(x_25) == 0) { -lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; size_t x_35; size_t x_36; lean_object* x_37; uint8_t x_38; -x_28 = lean_ctor_get(x_27, 0); -lean_inc(x_28); -x_29 = lean_ctor_get(x_27, 1); -lean_inc(x_29); -lean_dec(x_27); -x_30 = l_Lean_Elab_Structural_Positions_numIndices(x_2); -x_31 = l_Lean_Elab_Structural_inferBRecOnFTypes___closed__2; -x_32 = lean_mk_array(x_30, x_31); -x_33 = l_Array_toSubarray___rarg(x_2, x_11, x_9); -x_34 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_34, 0, x_33); -lean_ctor_set(x_34, 1, x_32); -x_35 = lean_array_size(x_28); -x_36 = 0; -x_37 = l_Array_forInUnsafe_loop___at_Lean_Elab_Structural_inferBRecOnFTypes___spec__2(x_28, x_35, x_36, x_34, x_4, x_5, x_6, x_7, x_29); +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; size_t x_34; size_t x_35; lean_object* x_36; uint8_t x_37; +x_26 = lean_ctor_get(x_25, 0); +lean_inc(x_26); +x_27 = lean_ctor_get(x_25, 1); +lean_inc(x_27); +lean_dec(x_25); +x_28 = l_Lean_Elab_Structural_Positions_numIndices(x_2); +x_29 = l_Lean_Elab_Structural_inferBRecOnFTypes___closed__2; +x_30 = lean_mk_array(x_28, x_29); +x_31 = lean_unsigned_to_nat(0u); +x_32 = l_Array_toSubarray___rarg(x_2, x_31, x_9); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_30); +x_34 = lean_array_size(x_26); +x_35 = 0; +x_36 = l_Array_forInUnsafe_loop___at_Lean_Elab_Structural_inferBRecOnFTypes___spec__2(x_26, x_34, x_35, x_33, x_4, x_5, x_6, x_7, x_27); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_28); -x_38 = !lean_is_exclusive(x_37); -if (x_38 == 0) +lean_dec(x_26); +x_37 = !lean_is_exclusive(x_36); +if (x_37 == 0) { -lean_object* x_39; lean_object* x_40; -x_39 = lean_ctor_get(x_37, 0); -x_40 = lean_ctor_get(x_39, 1); -lean_inc(x_40); -lean_dec(x_39); -lean_ctor_set(x_37, 0, x_40); -return x_37; +lean_object* x_38; lean_object* x_39; +x_38 = lean_ctor_get(x_36, 0); +x_39 = lean_ctor_get(x_38, 1); +lean_inc(x_39); +lean_dec(x_38); +lean_ctor_set(x_36, 0, x_39); +return x_36; } else { -lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_41 = lean_ctor_get(x_37, 0); -x_42 = lean_ctor_get(x_37, 1); -lean_inc(x_42); +lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_40 = lean_ctor_get(x_36, 0); +x_41 = lean_ctor_get(x_36, 1); lean_inc(x_41); -lean_dec(x_37); -x_43 = lean_ctor_get(x_41, 1); -lean_inc(x_43); -lean_dec(x_41); -x_44 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_44, 0, x_43); -lean_ctor_set(x_44, 1, x_42); -return x_44; +lean_inc(x_40); +lean_dec(x_36); +x_42 = lean_ctor_get(x_40, 1); +lean_inc(x_42); +lean_dec(x_40); +x_43 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_43, 0, x_42); +lean_ctor_set(x_43, 1, x_41); +return x_43; } } else { -uint8_t x_45; +uint8_t x_44; lean_dec(x_9); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); -x_45 = !lean_is_exclusive(x_27); -if (x_45 == 0) +x_44 = !lean_is_exclusive(x_25); +if (x_44 == 0) { -return x_27; +return x_25; } else { -lean_object* x_46; lean_object* x_47; lean_object* x_48; -x_46 = lean_ctor_get(x_27, 0); -x_47 = lean_ctor_get(x_27, 1); -lean_inc(x_47); +lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_45 = lean_ctor_get(x_25, 0); +x_46 = lean_ctor_get(x_25, 1); lean_inc(x_46); -lean_dec(x_27); -x_48 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_48, 0, x_46); -lean_ctor_set(x_48, 1, x_47); -return x_48; +lean_inc(x_45); +lean_dec(x_25); +x_47 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_47, 0, x_45); +lean_ctor_set(x_47, 1, x_46); +return x_47; } } } else { -uint8_t x_49; -lean_dec(x_15); +uint8_t x_48; +lean_dec(x_10); lean_dec(x_9); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); -x_49 = !lean_is_exclusive(x_17); -if (x_49 == 0) +x_48 = !lean_is_exclusive(x_15); +if (x_48 == 0) { -return x_17; +return x_15; } else { -lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_50 = lean_ctor_get(x_17, 0); -x_51 = lean_ctor_get(x_17, 1); -lean_inc(x_51); +lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_49 = lean_ctor_get(x_15, 0); +x_50 = lean_ctor_get(x_15, 1); lean_inc(x_50); -lean_dec(x_17); -x_52 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_52, 0, x_50); -lean_ctor_set(x_52, 1, x_51); -return x_52; +lean_inc(x_49); +lean_dec(x_15); +x_51 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_51, 0, x_49); +lean_ctor_set(x_51, 1, x_50); +return x_51; +} +} +} +else +{ +uint8_t x_52; +lean_dec(x_12); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +x_52 = !lean_is_exclusive(x_13); +if (x_52 == 0) +{ +return x_13; +} +else +{ +lean_object* x_53; lean_object* x_54; lean_object* x_55; +x_53 = lean_ctor_get(x_13, 0); +x_54 = lean_ctor_get(x_13, 1); +lean_inc(x_54); +lean_inc(x_53); +lean_dec(x_13); +x_55 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_55, 0, x_53); +lean_ctor_set(x_55, 1, x_54); +return x_55; } } } @@ -32557,34 +32302,32 @@ l_Lean_Elab_Structural_Positions_mapMwith___at___private_Lean_Elab_PreDefinition lean_mark_persistent(l_Lean_Elab_Structural_Positions_mapMwith___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__4___closed__8); l_Lean_Elab_Structural_Positions_mapMwith___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__4___closed__9 = _init_l_Lean_Elab_Structural_Positions_mapMwith___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__4___closed__9(); lean_mark_persistent(l_Lean_Elab_Structural_Positions_mapMwith___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__4___closed__9); -l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg___closed__1 = _init_l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg___closed__1(); -lean_mark_persistent(l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg___closed__1); -l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2___closed__1 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2___closed__1(); -lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2___closed__1); -l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2___closed__2 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2___closed__2(); -lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2___closed__2); -l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__1 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__1(); -lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__1); -l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__2 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__2(); -lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__2); -l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__3 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__3(); -lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__3); -l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__4 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__4(); -lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__4); -l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__5 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__5(); -lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__5); -l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4___closed__1 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4___closed__1(); -lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4___closed__1); -l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4___closed__2 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4___closed__2(); -lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4___closed__2); -l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5___closed__1 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5___closed__1(); -lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5___closed__1); -l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5___closed__2 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5___closed__2(); -lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5___closed__2); -l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___closed__1 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___closed__1(); -lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___closed__1); -l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___closed__2 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___closed__2(); -lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___closed__2); +l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2___closed__1 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2___closed__1); +l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2___closed__2 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2___closed__2(); +lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2___closed__2); +l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__1 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__1); +l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__2 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__2(); +lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__2); +l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__3 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__3(); +lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__3); +l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__4 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__4(); +lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__4); +l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__5 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__5(); +lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__5); +l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4___closed__1 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4___closed__1(); +lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4___closed__1); +l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4___closed__2 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4___closed__2(); +lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4___closed__2); +l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5___closed__1 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5___closed__1(); +lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5___closed__1); +l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5___closed__2 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5___closed__2(); +lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5___closed__2); +l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___closed__1 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___closed__1(); +lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___closed__1); +l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___closed__2 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___closed__2(); +lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___closed__2); l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___rarg___closed__1 = _init_l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___rarg___closed__1(); lean_mark_persistent(l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___rarg___closed__1); l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___rarg___closed__2 = _init_l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___rarg___closed__2(); @@ -32613,6 +32356,8 @@ l_List_forIn_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Le lean_mark_persistent(l_List_forIn_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__14___closed__4); l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__1 = _init_l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__1(); lean_mark_persistent(l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__1); +l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__2 = _init_l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__2(); +lean_mark_persistent(l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__2); l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___closed__1 = _init_l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___closed__1(); lean_mark_persistent(l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___closed__1); l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__22___closed__1 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__22___closed__1(); diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/Structural/FindRecArg.c b/stage0/stdlib/Lean/Elab/PreDefinition/Structural/FindRecArg.c index 97b4a2400d9e..1da398428595 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/Structural/FindRecArg.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/Structural/FindRecArg.c @@ -135,7 +135,6 @@ static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Structural_tryAllArg LEAN_EXPORT lean_object* l_Lean_Elab_Structural_prettyRecArg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Structural_inductiveGroups(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Structural_getRecArgInfo___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__31; LEAN_EXPORT lean_object* l_Lean_Elab_Structural_tryAllArgs___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Structural_tryAllArgs___spec__9___rarg___closed__7; @@ -241,7 +240,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_FindRecA LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Structural_tryAllArgs___spec__8___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_PersistentArray_anyM___at___private_Lean_Elab_PreDefinition_Structural_FindRecArg_0__Lean_Elab_Structural_hasBadIndexDep_x3f___spec__13(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Structural_tryAllArgs___rarg___lambda__4___closed__3; -static lean_object* l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__30; static lean_object* l_Lean_Elab_Structural_prettyParam___closed__2; lean_object* l_Lean_LocalDecl_fvarId(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Structural_tryAllArgs___spec__8___rarg___closed__4; @@ -5278,7 +5276,7 @@ static lean_object* _init_l_Lean_Elab_Structural_getRecArgInfo___lambda__1___clo _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked(" its type ", 10, 10); +x_1 = lean_mk_string_unchecked("its type ", 9, 9); return x_1; } } @@ -5410,7 +5408,7 @@ static lean_object* _init_l_Lean_Elab_Structural_getRecArgInfo___lambda__1___clo _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("its type ", 9, 9); +x_1 = lean_mk_string_unchecked(" is an inductive family", 23, 23); return x_1; } } @@ -5427,7 +5425,7 @@ static lean_object* _init_l_Lean_Elab_Structural_getRecArgInfo___lambda__1___clo _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked(" is an inductive family", 23, 23); +x_1 = lean_mk_string_unchecked("\nand index", 10, 10); return x_1; } } @@ -5444,7 +5442,7 @@ static lean_object* _init_l_Lean_Elab_Structural_getRecArgInfo___lambda__1___clo _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("\nand index", 10, 10); +x_1 = lean_mk_string_unchecked("\ndepends on the non index", 25, 25); return x_1; } } @@ -5461,7 +5459,7 @@ static lean_object* _init_l_Lean_Elab_Structural_getRecArgInfo___lambda__1___clo _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("\ndepends on the non index", 25, 25); +x_1 = lean_mk_string_unchecked(" is an inductive family and indices are not variables", 53, 53); return x_1; } } @@ -5478,7 +5476,7 @@ static lean_object* _init_l_Lean_Elab_Structural_getRecArgInfo___lambda__1___clo _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked(" is an inductive family and indices are not variables", 53, 53); +x_1 = lean_mk_string_unchecked(" is a reflexive inductive, but ", 31, 31); return x_1; } } @@ -5495,7 +5493,7 @@ static lean_object* _init_l_Lean_Elab_Structural_getRecArgInfo___lambda__1___clo _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked(" is a reflexive inductive, but ", 31, 31); +x_1 = lean_mk_string_unchecked(" does not exist and it is not an inductive predicate", 52, 52); return x_1; } } @@ -5508,23 +5506,6 @@ x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__30() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked(" does not exist and it is not an inductive predicate", 52, 52); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__31() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__30; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} LEAN_EXPORT lean_object* l_Lean_Elab_Structural_getRecArgInfo___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { @@ -5668,11 +5649,11 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); x_215 = l_Lean_MessageData_ofName(x_30); -x_216 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__19; +x_216 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__4; x_217 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_217, 0, x_216); lean_ctor_set(x_217, 1, x_215); -x_218 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__29; +x_218 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__27; x_219 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_219, 0, x_217); lean_ctor_set(x_219, 1, x_218); @@ -5680,7 +5661,7 @@ x_220 = l_Lean_MessageData_ofName(x_32); x_221 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_221, 0, x_219); lean_ctor_set(x_221, 1, x_220); -x_222 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__31; +x_222 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__29; x_223 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_223, 0, x_221); lean_ctor_set(x_223, 1, x_222); @@ -5855,11 +5836,11 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); x_200 = l_Lean_MessageData_ofName(x_30); -x_201 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__19; +x_201 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__4; x_202 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_202, 0, x_201); lean_ctor_set(x_202, 1, x_200); -x_203 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__27; +x_203 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__25; x_204 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_204, 0, x_202); lean_ctor_set(x_204, 1, x_203); @@ -6172,11 +6153,11 @@ lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; x_144 = lean_ctor_get(x_141, 0); x_145 = lean_ctor_get(x_141, 1); x_146 = l_Lean_MessageData_ofName(x_30); -x_147 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__19; +x_147 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__4; lean_ctor_set_tag(x_141, 7); lean_ctor_set(x_141, 1, x_146); lean_ctor_set(x_141, 0, x_147); -x_148 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__21; +x_148 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__19; x_149 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_149, 0, x_141); lean_ctor_set(x_149, 1, x_148); @@ -6184,7 +6165,7 @@ x_150 = l_Lean_indentExpr(x_14); x_151 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_151, 0, x_149); lean_ctor_set(x_151, 1, x_150); -x_152 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__23; +x_152 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__21; x_153 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_153, 0, x_151); lean_ctor_set(x_153, 1, x_152); @@ -6192,7 +6173,7 @@ x_154 = l_Lean_indentExpr(x_144); x_155 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_155, 0, x_153); lean_ctor_set(x_155, 1, x_154); -x_156 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__25; +x_156 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__23; x_157 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_157, 0, x_155); lean_ctor_set(x_157, 1, x_156); @@ -6220,11 +6201,11 @@ lean_inc(x_164); lean_inc(x_163); lean_dec(x_141); x_165 = l_Lean_MessageData_ofName(x_30); -x_166 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__19; +x_166 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__4; x_167 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_167, 0, x_166); lean_ctor_set(x_167, 1, x_165); -x_168 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__21; +x_168 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__19; x_169 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_169, 0, x_167); lean_ctor_set(x_169, 1, x_168); @@ -6232,7 +6213,7 @@ x_170 = l_Lean_indentExpr(x_14); x_171 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_171, 0, x_169); lean_ctor_set(x_171, 1, x_170); -x_172 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__23; +x_172 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__21; x_173 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_173, 0, x_171); lean_ctor_set(x_173, 1, x_172); @@ -6240,7 +6221,7 @@ x_174 = l_Lean_indentExpr(x_163); x_175 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_175, 0, x_173); lean_ctor_set(x_175, 1, x_174); -x_176 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__25; +x_176 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__23; x_177 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_177, 0, x_175); lean_ctor_set(x_177, 1, x_176); @@ -17276,10 +17257,6 @@ l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__28 = _init_l_Lean_Ela lean_mark_persistent(l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__28); l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__29 = _init_l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__29(); lean_mark_persistent(l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__29); -l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__30 = _init_l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__30(); -lean_mark_persistent(l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__30); -l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__31 = _init_l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__31(); -lean_mark_persistent(l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__31); l_Lean_Elab_Structural_getRecArgInfo___lambda__2___closed__1 = _init_l_Lean_Elab_Structural_getRecArgInfo___lambda__2___closed__1(); lean_mark_persistent(l_Lean_Elab_Structural_getRecArgInfo___lambda__2___closed__1); l_Lean_Elab_Structural_getRecArgInfo___lambda__2___closed__2 = _init_l_Lean_Elab_Structural_getRecArgInfo___lambda__2___closed__2(); diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/Structural/Main.c b/stage0/stdlib/Lean/Elab/PreDefinition/Structural/Main.c index 5caddcbec9bc..a63bacb44620 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/Structural/Main.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/Structural/Main.c @@ -24,7 +24,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Structural_getMutualFixedPrefix(lean_object lean_object* l_Lean_Elab_Structural_mkBrecOnApp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__3___closed__4; lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withLocalContextImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Elab_instInhabitedPreDefinition; LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_inferRecArgPos___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Structural_getMutualFixedPrefix___spec__14___lambda__3___closed__2; @@ -44,7 +44,6 @@ static lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_ LEAN_EXPORT lean_object* l_Lean_Meta_visitLambda_visit___at_Lean_Elab_Structural_getMutualFixedPrefix___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at_Lean_Elab_Structural_getMutualFixedPrefix___spec__13___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__16(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Elab_Structural_getMutualFixedPrefix___spec__7___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_inferRecArgPos___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_lambdaTelescope___at___private_Lean_Meta_Eqns_0__Lean_Meta_mkSimpleEqThm___spec__1___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -154,6 +153,7 @@ lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_setEnv___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_inferRecArgPos___spec__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_inferRecArgPos___lambda__5___closed__4; LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_inferRecArgPos___spec__20(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_lambdaBoundedTelescope___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_inferRecArgPos___spec__15___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_inferRecArgPos___spec__26___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -226,7 +226,8 @@ lean_object* l_Lean_Elab_Structural_run___rarg(lean_object*, lean_object*, lean_ LEAN_EXPORT lean_object* l_Lean_Elab_Structural_getMutualFixedPrefix___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_ST_Prim_Ref_modifyGetUnsafe___rarg___boxed(lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_levelZero; -LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__8; +LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_abstractNestedProofs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Structural_reportTermArg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_instInhabitedExpr; @@ -278,7 +279,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_forEachExpr_x27_visit___at_Lean_Elab_Struct static lean_object* l_Lean_Elab_Structural_getMutualFixedPrefix___lambda__2___closed__2; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Structural_structuralRecursion___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Structural_getMutualFixedPrefix___spec__14___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__3___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_getFixedPrefix(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -415,7 +415,7 @@ uint8_t lean_usize_dec_lt(size_t, size_t); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_inferRecArgPos___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_inferRecArgPos___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_inferRecArgPos___spec__8(lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkLambdaFVars(lean_object*, lean_object*, uint8_t, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__13___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__14(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_forEachExpr_x27___at_Lean_Elab_Structural_getMutualFixedPrefix___spec__3___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -425,8 +425,10 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefi static lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__4___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at_Lean_Elab_Structural_getMutualFixedPrefix___spec__13___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__5(lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Structural_getMutualFixedPrefix___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6(lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__9; +LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6(lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Split_0__Lean_Meta_Split_generalizeMatchDiscrs___spec__1(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_visitLambda_visit___at_Lean_Elab_Structural_getMutualFixedPrefix___spec__6___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -434,6 +436,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__ lean_object* lean_array_uset(lean_object*, size_t, lean_object*); lean_object* l_ReaderT_bind___at___private_Lean_Elab_PreDefinition_Structural_IndPred_0__Lean_Elab_Structural_replaceIndPredRecApp___spec__8___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_MessageData_ofName(lean_object*); lean_object* lean_expr_instantiate1(lean_object*, lean_object*); lean_object* l___private_Init_Data_Repr_0__Nat_reprFast(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_getFixedPrefix___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -6581,100 +6584,100 @@ return x_31; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { -lean_object* x_17; uint8_t x_18; -x_17 = lean_unsigned_to_nat(0u); -x_18 = lean_nat_dec_eq(x_7, x_17); -if (x_18 == 0) +lean_object* x_16; uint8_t x_17; +x_16 = lean_unsigned_to_nat(0u); +x_17 = lean_nat_dec_eq(x_6, x_16); +if (x_17 == 0) { -lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_19 = lean_unsigned_to_nat(1u); -x_20 = lean_nat_sub(x_7, x_19); -lean_dec(x_7); -x_21 = lean_array_fget(x_6, x_8); -x_22 = lean_ctor_get(x_21, 0); +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_18 = lean_unsigned_to_nat(1u); +x_19 = lean_nat_sub(x_6, x_18); +lean_dec(x_6); +x_20 = lean_array_fget(x_5, x_7); +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_20, 1); lean_inc(x_22); -x_23 = lean_ctor_get(x_21, 1); -lean_inc(x_23); -lean_dec(x_21); -lean_inc(x_15); +lean_dec(x_20); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -lean_inc(x_5); +lean_inc(x_11); lean_inc(x_4); -lean_inc(x_8); lean_inc(x_3); -x_24 = l_Lean_Elab_Structural_mkBrecOnApp(x_3, x_8, x_4, x_5, x_22, x_23, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_24) == 0) +lean_inc(x_7); +lean_inc(x_1); +x_23 = l_Lean_Elab_Structural_mkBrecOnApp(x_1, x_7, x_3, x_4, x_21, x_22, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_23) == 0) { -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_25 = lean_ctor_get(x_24, 0); +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_23, 1); lean_inc(x_25); -x_26 = lean_ctor_get(x_24, 1); -lean_inc(x_26); -lean_dec(x_24); -x_27 = lean_nat_add(x_8, x_19); -lean_dec(x_8); -x_28 = lean_array_push(x_10, x_25); -x_7 = x_20; -x_8 = x_27; -x_9 = lean_box(0); -x_10 = x_28; -x_16 = x_26; +lean_dec(x_23); +x_26 = lean_nat_add(x_7, x_18); +lean_dec(x_7); +x_27 = lean_array_push(x_9, x_24); +x_6 = x_19; +x_7 = x_26; +x_8 = lean_box(0); +x_9 = x_27; +x_15 = x_25; goto _start; } else { -uint8_t x_30; -lean_dec(x_20); -lean_dec(x_15); +uint8_t x_29; +lean_dec(x_19); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); -lean_dec(x_10); -lean_dec(x_8); -lean_dec(x_5); +lean_dec(x_11); +lean_dec(x_9); +lean_dec(x_7); lean_dec(x_4); lean_dec(x_3); -x_30 = !lean_is_exclusive(x_24); -if (x_30 == 0) +lean_dec(x_1); +x_29 = !lean_is_exclusive(x_23); +if (x_29 == 0) { -return x_24; +return x_23; } else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_31 = lean_ctor_get(x_24, 0); -x_32 = lean_ctor_get(x_24, 1); -lean_inc(x_32); +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_23, 0); +x_31 = lean_ctor_get(x_23, 1); lean_inc(x_31); -lean_dec(x_24); -x_33 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_33, 0, x_31); -lean_ctor_set(x_33, 1, x_32); -return x_33; +lean_inc(x_30); +lean_dec(x_23); +x_32 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_31); +return x_32; } } } else { -lean_object* x_34; -lean_dec(x_15); +lean_object* x_33; lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); -lean_dec(x_8); +lean_dec(x_11); lean_dec(x_7); -lean_dec(x_5); +lean_dec(x_6); lean_dec(x_4); lean_dec(x_3); -x_34 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_34, 0, x_10); -lean_ctor_set(x_34, 1, x_16); -return x_34; +lean_dec(x_1); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_9); +lean_ctor_set(x_33, 1, x_15); +return x_33; } } } @@ -7042,113 +7045,113 @@ lean_inc(x_2); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, size_t x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_17 = lean_array_get_size(x_1); -x_18 = lean_mk_empty_array_with_capacity(x_17); -x_19 = lean_unsigned_to_nat(0u); -lean_inc(x_15); -lean_inc(x_14); +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_15 = lean_array_get_size(x_1); +x_16 = lean_mk_empty_array_with_capacity(x_15); +x_17 = lean_unsigned_to_nat(0u); lean_inc(x_13); lean_inc(x_12); -x_20 = l_Array_mapIdxM_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__10(x_2, x_3, x_4, x_5, x_6, x_1, x_17, x_19, lean_box(0), x_18, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_20) == 0) +lean_inc(x_11); +lean_inc(x_10); +x_18 = l_Array_mapFinIdxM_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__10(x_2, x_1, x_3, x_4, x_1, x_15, x_17, lean_box(0), x_16, x_9, x_10, x_11, x_12, x_13, x_14); +if (lean_obj_tag(x_18) == 0) { -lean_object* x_21; lean_object* x_22; size_t x_23; lean_object* x_24; -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_20, 1); -lean_inc(x_22); -lean_dec(x_20); -x_23 = lean_array_size(x_21); -x_24 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__11(x_7, x_23, x_8, x_21, x_11, x_12, x_13, x_14, x_15, x_22); -lean_dec(x_15); -lean_dec(x_14); +lean_object* x_19; lean_object* x_20; size_t x_21; lean_object* x_22; +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +x_20 = lean_ctor_get(x_18, 1); +lean_inc(x_20); +lean_dec(x_18); +x_21 = lean_array_size(x_19); +x_22 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__11(x_5, x_21, x_6, x_19, x_9, x_10, x_11, x_12, x_13, x_20); lean_dec(x_13); lean_dec(x_12); -if (lean_obj_tag(x_24) == 0) +lean_dec(x_11); +lean_dec(x_10); +if (lean_obj_tag(x_22) == 0) { -uint8_t x_25; -x_25 = !lean_is_exclusive(x_24); -if (x_25 == 0) +uint8_t x_23; +x_23 = !lean_is_exclusive(x_22); +if (x_23 == 0) { -lean_object* x_26; lean_object* x_27; size_t x_28; lean_object* x_29; -x_26 = lean_ctor_get(x_24, 0); -x_27 = l_Array_zip___rarg(x_9, x_26); -lean_dec(x_26); -x_28 = lean_array_size(x_27); -x_29 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__12(x_28, x_8, x_27); -lean_ctor_set(x_24, 0, x_29); -return x_24; +lean_object* x_24; lean_object* x_25; size_t x_26; lean_object* x_27; +x_24 = lean_ctor_get(x_22, 0); +x_25 = l_Array_zip___rarg(x_7, x_24); +lean_dec(x_24); +x_26 = lean_array_size(x_25); +x_27 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__12(x_26, x_6, x_25); +lean_ctor_set(x_22, 0, x_27); +return x_22; } else { -lean_object* x_30; lean_object* x_31; lean_object* x_32; size_t x_33; lean_object* x_34; lean_object* x_35; -x_30 = lean_ctor_get(x_24, 0); -x_31 = lean_ctor_get(x_24, 1); -lean_inc(x_31); -lean_inc(x_30); -lean_dec(x_24); -x_32 = l_Array_zip___rarg(x_9, x_30); -lean_dec(x_30); -x_33 = lean_array_size(x_32); -x_34 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__12(x_33, x_8, x_32); -x_35 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_35, 0, x_34); -lean_ctor_set(x_35, 1, x_31); -return x_35; +lean_object* x_28; lean_object* x_29; lean_object* x_30; size_t x_31; lean_object* x_32; lean_object* x_33; +x_28 = lean_ctor_get(x_22, 0); +x_29 = lean_ctor_get(x_22, 1); +lean_inc(x_29); +lean_inc(x_28); +lean_dec(x_22); +x_30 = l_Array_zip___rarg(x_7, x_28); +lean_dec(x_28); +x_31 = lean_array_size(x_30); +x_32 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__12(x_31, x_6, x_30); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_29); +return x_33; } } else { -uint8_t x_36; -x_36 = !lean_is_exclusive(x_24); -if (x_36 == 0) +uint8_t x_34; +x_34 = !lean_is_exclusive(x_22); +if (x_34 == 0) { -return x_24; +return x_22; } else { -lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_37 = lean_ctor_get(x_24, 0); -x_38 = lean_ctor_get(x_24, 1); -lean_inc(x_38); -lean_inc(x_37); -lean_dec(x_24); -x_39 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_39, 0, x_37); -lean_ctor_set(x_39, 1, x_38); -return x_39; +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_22, 0); +x_36 = lean_ctor_get(x_22, 1); +lean_inc(x_36); +lean_inc(x_35); +lean_dec(x_22); +x_37 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +return x_37; } } } else { -uint8_t x_40; -lean_dec(x_15); -lean_dec(x_14); +uint8_t x_38; lean_dec(x_13); lean_dec(x_12); -lean_dec(x_7); -x_40 = !lean_is_exclusive(x_20); -if (x_40 == 0) +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_5); +x_38 = !lean_is_exclusive(x_18); +if (x_38 == 0) { -return x_20; +return x_18; } else { -lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_ctor_get(x_20, 0); -x_42 = lean_ctor_get(x_20, 1); -lean_inc(x_42); -lean_inc(x_41); -lean_dec(x_20); -x_43 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_43, 0, x_41); -lean_ctor_set(x_43, 1, x_42); -return x_43; +lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = lean_ctor_get(x_18, 0); +x_40 = lean_ctor_get(x_18, 1); +lean_inc(x_40); +lean_inc(x_39); +lean_dec(x_18); +x_41 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_41, 0, x_39); +lean_ctor_set(x_41, 1, x_40); +return x_41; } } } @@ -7201,7 +7204,6 @@ lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_4); -lean_inc(x_3); x_21 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__9(x_3, x_4, x_20, x_5, x_19, x_12, x_13, x_14, x_15, x_16, x_17); if (lean_obj_tag(x_21) == 0) { @@ -7225,9 +7227,8 @@ x_27 = lean_ctor_get(x_24, 1); lean_inc(x_27); lean_dec(x_24); x_28 = lean_box(0); -x_29 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__2(x_7, x_3, x_1, x_4, x_8, x_22, x_9, x_5, x_10, x_28, x_12, x_13, x_14, x_15, x_16, x_27); +x_29 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__2(x_7, x_4, x_8, x_22, x_9, x_5, x_10, x_28, x_12, x_13, x_14, x_15, x_16, x_27); lean_dec(x_12); -lean_dec(x_3); return x_29; } else @@ -7259,10 +7260,9 @@ lean_inc(x_41); x_42 = lean_ctor_get(x_40, 1); lean_inc(x_42); lean_dec(x_40); -x_43 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__2(x_7, x_3, x_1, x_4, x_8, x_22, x_9, x_5, x_10, x_41, x_12, x_13, x_14, x_15, x_16, x_42); +x_43 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__2(x_7, x_4, x_8, x_22, x_9, x_5, x_10, x_41, x_12, x_13, x_14, x_15, x_16, x_42); lean_dec(x_12); lean_dec(x_41); -lean_dec(x_3); return x_43; } else @@ -7290,10 +7290,9 @@ lean_inc(x_54); x_55 = lean_ctor_get(x_53, 1); lean_inc(x_55); lean_dec(x_53); -x_56 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__2(x_7, x_3, x_1, x_4, x_8, x_22, x_9, x_5, x_10, x_54, x_12, x_13, x_14, x_15, x_16, x_55); +x_56 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__2(x_7, x_4, x_8, x_22, x_9, x_5, x_10, x_54, x_12, x_13, x_14, x_15, x_16, x_55); lean_dec(x_12); lean_dec(x_54); -lean_dec(x_3); return x_56; } } @@ -7310,7 +7309,6 @@ lean_dec(x_9); lean_dec(x_8); lean_dec(x_6); lean_dec(x_4); -lean_dec(x_3); x_57 = !lean_is_exclusive(x_21); if (x_57 == 0) { @@ -7739,7 +7737,7 @@ static lean_object* _init_l___private_Lean_Elab_PreDefinition_Structural_Main_0_ _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("positions: ", 11, 11); +x_1 = lean_mk_string_unchecked("assignments of type formers of ", 31, 31); return x_1; } } @@ -7752,92 +7750,126 @@ x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +static lean_object* _init_l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__8() { _start: { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; -x_14 = l_Lean_InductiveVal_numTypeFormers(x_1); -x_15 = l_Array_range(x_14); -x_16 = l_Lean_Elab_Structural_instInhabitedRecArgInfo; -x_17 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__1; -x_18 = l_Lean_Elab_Structural_Positions_groupAndSort___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__4(x_16, x_17, x_2, x_15); -x_19 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__5; -x_20 = l_Lean_isTracingEnabledFor___at___private_Lean_Elab_PreDefinition_Structural_IndPred_0__Lean_Elab_Structural_replaceIndPredRecApp___spec__2(x_19, x_8, x_9, x_10, x_11, x_12, x_13); -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -x_22 = lean_unbox(x_21); -lean_dec(x_21); -if (x_22 == 0) +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" to functions: ", 15, 15); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__9() { +_start: { -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_20, 1); -lean_inc(x_23); -lean_dec(x_20); -x_24 = lean_box(0); -x_25 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__5(x_2, x_3, x_4, x_19, x_18, x_5, x_6, x_24, x_8, x_9, x_10, x_11, x_12, x_23); -return x_25; +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__8; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_15 = l_Lean_InductiveVal_numTypeFormers(x_1); +x_16 = l_Array_range(x_15); +x_17 = l_Lean_Elab_Structural_instInhabitedRecArgInfo; +x_18 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__1; +x_19 = l_Lean_Elab_Structural_Positions_groupAndSort___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__4(x_17, x_18, x_2, x_16); +x_20 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__5; +x_21 = l_Lean_isTracingEnabledFor___at___private_Lean_Elab_PreDefinition_Structural_IndPred_0__Lean_Elab_Structural_replaceIndPredRecApp___spec__2(x_20, x_9, x_10, x_11, x_12, x_13, x_14); +x_22 = lean_ctor_get(x_21, 0); +lean_inc(x_22); +x_23 = lean_unbox(x_22); +lean_dec(x_22); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; +lean_dec(x_7); +x_24 = lean_ctor_get(x_21, 1); +lean_inc(x_24); +lean_dec(x_21); +x_25 = lean_box(0); +x_26 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__5(x_2, x_3, x_4, x_20, x_19, x_5, x_6, x_25, x_9, x_10, x_11, x_12, x_13, x_24); +return x_26; } else { -uint8_t x_26; -x_26 = !lean_is_exclusive(x_20); -if (x_26 == 0) +uint8_t x_27; +x_27 = !lean_is_exclusive(x_21); +if (x_27 == 0) { -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_27 = lean_ctor_get(x_20, 1); -x_28 = lean_ctor_get(x_20, 0); -lean_dec(x_28); -lean_inc(x_18); -x_29 = lean_array_to_list(x_18); -x_30 = lean_box(0); -x_31 = l_List_mapTR_loop___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__16(x_29, x_30); -x_32 = l_Lean_MessageData_ofList(x_31); -x_33 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__7; -lean_ctor_set_tag(x_20, 7); -lean_ctor_set(x_20, 1, x_32); -lean_ctor_set(x_20, 0, x_33); -x_34 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__3___closed__4; -x_35 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_35, 0, x_20); -lean_ctor_set(x_35, 1, x_34); -x_36 = l_Lean_addTrace___at___private_Lean_Elab_PreDefinition_Structural_IndPred_0__Lean_Elab_Structural_replaceIndPredRecApp___spec__3(x_19, x_35, x_8, x_9, x_10, x_11, x_12, x_27); -x_37 = lean_ctor_get(x_36, 0); -lean_inc(x_37); -x_38 = lean_ctor_get(x_36, 1); -lean_inc(x_38); -lean_dec(x_36); -x_39 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__5(x_2, x_3, x_4, x_19, x_18, x_5, x_6, x_37, x_8, x_9, x_10, x_11, x_12, x_38); -lean_dec(x_37); -return x_39; +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_28 = lean_ctor_get(x_21, 1); +x_29 = lean_ctor_get(x_21, 0); +lean_dec(x_29); +x_30 = l_Lean_MessageData_ofName(x_7); +x_31 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__7; +lean_ctor_set_tag(x_21, 7); +lean_ctor_set(x_21, 1, x_30); +lean_ctor_set(x_21, 0, x_31); +x_32 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__9; +x_33 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_33, 0, x_21); +lean_ctor_set(x_33, 1, x_32); +lean_inc(x_19); +x_34 = lean_array_to_list(x_19); +x_35 = lean_box(0); +x_36 = l_List_mapTR_loop___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__16(x_34, x_35); +x_37 = l_Lean_MessageData_ofList(x_36); +x_38 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_38, 0, x_33); +lean_ctor_set(x_38, 1, x_37); +x_39 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__3___closed__4; +x_40 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +x_41 = l_Lean_addTrace___at___private_Lean_Elab_PreDefinition_Structural_IndPred_0__Lean_Elab_Structural_replaceIndPredRecApp___spec__3(x_20, x_40, x_9, x_10, x_11, x_12, x_13, x_28); +x_42 = lean_ctor_get(x_41, 0); +lean_inc(x_42); +x_43 = lean_ctor_get(x_41, 1); +lean_inc(x_43); +lean_dec(x_41); +x_44 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__5(x_2, x_3, x_4, x_20, x_19, x_5, x_6, x_42, x_9, x_10, x_11, x_12, x_13, x_43); +lean_dec(x_42); +return x_44; } else { -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_40 = lean_ctor_get(x_20, 1); -lean_inc(x_40); -lean_dec(x_20); -lean_inc(x_18); -x_41 = lean_array_to_list(x_18); -x_42 = lean_box(0); -x_43 = l_List_mapTR_loop___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__16(x_41, x_42); -x_44 = l_Lean_MessageData_ofList(x_43); -x_45 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__7; -x_46 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_46, 0, x_45); -lean_ctor_set(x_46, 1, x_44); -x_47 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__3___closed__4; +lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; +x_45 = lean_ctor_get(x_21, 1); +lean_inc(x_45); +lean_dec(x_21); +x_46 = l_Lean_MessageData_ofName(x_7); +x_47 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__7; x_48 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_48, 0, x_46); -lean_ctor_set(x_48, 1, x_47); -x_49 = l_Lean_addTrace___at___private_Lean_Elab_PreDefinition_Structural_IndPred_0__Lean_Elab_Structural_replaceIndPredRecApp___spec__3(x_19, x_48, x_8, x_9, x_10, x_11, x_12, x_40); -x_50 = lean_ctor_get(x_49, 0); -lean_inc(x_50); -x_51 = lean_ctor_get(x_49, 1); -lean_inc(x_51); -lean_dec(x_49); -x_52 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__5(x_2, x_3, x_4, x_19, x_18, x_5, x_6, x_50, x_8, x_9, x_10, x_11, x_12, x_51); -lean_dec(x_50); -return x_52; +lean_ctor_set(x_48, 0, x_47); +lean_ctor_set(x_48, 1, x_46); +x_49 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__9; +x_50 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_50, 0, x_48); +lean_ctor_set(x_50, 1, x_49); +lean_inc(x_19); +x_51 = lean_array_to_list(x_19); +x_52 = lean_box(0); +x_53 = l_List_mapTR_loop___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__16(x_51, x_52); +x_54 = l_Lean_MessageData_ofList(x_53); +x_55 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_55, 0, x_50); +lean_ctor_set(x_55, 1, x_54); +x_56 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__3___closed__4; +x_57 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_57, 0, x_55); +lean_ctor_set(x_57, 1, x_56); +x_58 = l_Lean_addTrace___at___private_Lean_Elab_PreDefinition_Structural_IndPred_0__Lean_Elab_Structural_replaceIndPredRecApp___spec__3(x_20, x_57, x_9, x_10, x_11, x_12, x_13, x_45); +x_59 = lean_ctor_get(x_58, 0); +lean_inc(x_59); +x_60 = lean_ctor_get(x_58, 1); +lean_inc(x_60); +lean_dec(x_58); +x_61 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__5(x_2, x_3, x_4, x_20, x_19, x_5, x_6, x_59, x_9, x_10, x_11, x_12, x_13, x_60); +lean_dec(x_59); +return x_61; } } } @@ -8386,6 +8418,7 @@ lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); +lean_inc(x_21); x_22 = l_Lean_Meta_isInductivePredicate(x_21, x_5, x_6, x_7, x_8, x_19); if (lean_obj_tag(x_22) == 0) { @@ -8402,7 +8435,7 @@ x_25 = lean_ctor_get(x_22, 1); lean_inc(x_25); lean_dec(x_22); x_26 = lean_box(0); -x_27 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6(x_18, x_3, x_13, x_11, x_2, x_1, x_26, x_4, x_5, x_6, x_7, x_8, x_25); +x_27 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6(x_18, x_3, x_13, x_11, x_2, x_1, x_21, x_26, x_4, x_5, x_6, x_7, x_8, x_25); lean_dec(x_1); lean_dec(x_13); lean_dec(x_18); @@ -8411,6 +8444,7 @@ return x_27; else { lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; +lean_dec(x_21); lean_dec(x_18); lean_dec(x_3); x_28 = lean_ctor_get(x_22, 1); @@ -8467,6 +8501,7 @@ return x_39; else { uint8_t x_40; +lean_dec(x_21); lean_dec(x_18); lean_dec(x_15); lean_dec(x_13); @@ -8680,16 +8715,15 @@ x_14 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_ return x_14; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { -lean_object* x_17; -x_17 = l_Array_mapIdxM_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__10(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_11); -lean_dec(x_6); +lean_object* x_16; +x_16 = l_Array_mapFinIdxM_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__10(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +lean_dec(x_10); +lean_dec(x_5); lean_dec(x_2); -lean_dec(x_1); -return x_17; +return x_16; } } LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { @@ -8730,20 +8764,18 @@ lean_dec(x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { -size_t x_17; lean_object* x_18; -x_17 = lean_unbox_usize(x_8); -lean_dec(x_8); -x_18 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_17, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_11); -lean_dec(x_10); +size_t x_15; lean_object* x_16; +x_15 = lean_unbox_usize(x_6); +lean_dec(x_6); +x_16 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__2(x_1, x_2, x_3, x_4, x_5, x_15, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); lean_dec(x_9); -lean_dec(x_3); -lean_dec(x_2); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_1); -return x_18; +return x_16; } } LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__3___boxed(lean_object** _args) { @@ -8806,18 +8838,18 @@ lean_dec(x_2); return x_16; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { -size_t x_14; lean_object* x_15; -x_14 = lean_unbox_usize(x_4); +size_t x_15; lean_object* x_16; +x_15 = lean_unbox_usize(x_4); lean_dec(x_4); -x_15 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6(x_1, x_2, x_3, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_7); +x_16 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6(x_1, x_2, x_3, x_15, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_8); lean_dec(x_6); lean_dec(x_3); lean_dec(x_1); -return x_15; +return x_16; } } LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { @@ -15918,6 +15950,10 @@ l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elim lean_mark_persistent(l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__6); l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__7 = _init_l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__7(); lean_mark_persistent(l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__7); +l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__8 = _init_l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__8(); +lean_mark_persistent(l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__8); +l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__9 = _init_l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__9(); +lean_mark_persistent(l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__9); l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__8___closed__1 = _init_l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__8___closed__1(); lean_mark_persistent(l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__8___closed__1); l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__8___closed__2 = _init_l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__8___closed__2(); diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/Structural/SmartUnfolding.c b/stage0/stdlib/Lean/Elab/PreDefinition/Structural/SmartUnfolding.c index b98f3ad63761..e3f05672380d 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/Structural/SmartUnfolding.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/Structural/SmartUnfolding.c @@ -17,6 +17,7 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Structural_addS LEAN_EXPORT lean_object* l_Lean_Elab_Structural_addSmartUnfoldingDefAux_visit___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_lambdaBoundedTelescope___at_Lean_Elab_Structural_addSmartUnfoldingDefAux_visit___spec__8___rarg(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_getConstInfo___at_Lean_Meta_mkConstWithFreshMVarLevels___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_mk_empty_array_with_capacity(lean_object*); lean_object* l_Lean_mkAppN(lean_object*, lean_object*); lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_lambdaBoundedTelescope___at_Lean_Elab_Structural_addSmartUnfoldingDefAux_visit___spec__8___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -67,6 +68,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at_Lean_Elab_Structural_addSm LEAN_EXPORT lean_object* l_Lean_Elab_Structural_addSmartUnfoldingDefAux_visit___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_levelZero; extern lean_object* l_Lean_instInhabitedExpr; +static lean_object* l_Lean_Elab_Structural_addSmartUnfoldingDefAux___closed__2; LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Elab_Structural_addSmartUnfoldingDefAux_visit___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_lengthTRAux___rarg(lean_object*, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); @@ -3467,20 +3469,31 @@ return x_10; static lean_object* _init_l_Lean_Elab_Structural_addSmartUnfoldingDefAux___closed__1() { _start: { -lean_object* x_1; uint8_t x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(0u); +x_2 = lean_mk_empty_array_with_capacity(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Structural_addSmartUnfoldingDefAux___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; uint8_t x_5; lean_object* x_6; lean_object* x_7; x_1 = lean_box(0); -x_2 = 0; +x_2 = lean_box(0); x_3 = 0; -x_4 = 2; -x_5 = l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Elab_Structural_addSmartUnfoldingDefAux_visit___spec__1___lambda__2___closed__1; -x_6 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_6, 0, x_1); -lean_ctor_set(x_6, 1, x_5); -lean_ctor_set_uint8(x_6, sizeof(void*)*2, x_2); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 1, x_3); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 2, x_4); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 3, x_3); -return x_6; +x_4 = 0; +x_5 = 0; +x_6 = l_Lean_Elab_Structural_addSmartUnfoldingDefAux___closed__1; +x_7 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_7, 0, x_2); +lean_ctor_set(x_7, 1, x_1); +lean_ctor_set(x_7, 2, x_6); +lean_ctor_set_uint8(x_7, sizeof(void*)*3, x_3); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 1, x_4); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 2, x_5); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 3, x_4); +return x_7; } } LEAN_EXPORT lean_object* l_Lean_Elab_Structural_addSmartUnfoldingDefAux(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { @@ -3530,7 +3543,7 @@ lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; x_25 = lean_ctor_get(x_15, 0); x_26 = l_Lean_Meta_smartUnfoldingSuffix; x_27 = l_Lean_Name_str___override(x_11, x_26); -x_28 = l_Lean_Elab_Structural_addSmartUnfoldingDefAux___closed__1; +x_28 = l_Lean_Elab_Structural_addSmartUnfoldingDefAux___closed__2; lean_ctor_set(x_1, 5, x_25); lean_ctor_set(x_1, 3, x_27); lean_ctor_set(x_1, 2, x_28); @@ -3547,7 +3560,7 @@ lean_inc(x_29); lean_dec(x_15); x_31 = l_Lean_Meta_smartUnfoldingSuffix; x_32 = l_Lean_Name_str___override(x_11, x_31); -x_33 = l_Lean_Elab_Structural_addSmartUnfoldingDefAux___closed__1; +x_33 = l_Lean_Elab_Structural_addSmartUnfoldingDefAux___closed__2; lean_ctor_set(x_1, 5, x_29); lean_ctor_set(x_1, 3, x_32); lean_ctor_set(x_1, 2, x_33); @@ -3606,7 +3619,7 @@ if (lean_is_exclusive(x_15)) { } x_42 = l_Lean_Meta_smartUnfoldingSuffix; x_43 = l_Lean_Name_str___override(x_11, x_42); -x_44 = l_Lean_Elab_Structural_addSmartUnfoldingDefAux___closed__1; +x_44 = l_Lean_Elab_Structural_addSmartUnfoldingDefAux___closed__2; x_45 = lean_alloc_ctor(0, 7, 1); lean_ctor_set(x_45, 0, x_8); lean_ctor_set(x_45, 1, x_10); @@ -3864,6 +3877,8 @@ l_Array_forInUnsafe_loop___at_Lean_Elab_Structural_addSmartUnfoldingDefAux_visit lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Structural_addSmartUnfoldingDefAux_visit___spec__9___lambda__3___closed__6); l_Lean_Elab_Structural_addSmartUnfoldingDefAux___closed__1 = _init_l_Lean_Elab_Structural_addSmartUnfoldingDefAux___closed__1(); lean_mark_persistent(l_Lean_Elab_Structural_addSmartUnfoldingDefAux___closed__1); +l_Lean_Elab_Structural_addSmartUnfoldingDefAux___closed__2 = _init_l_Lean_Elab_Structural_addSmartUnfoldingDefAux___closed__2(); +lean_mark_persistent(l_Lean_Elab_Structural_addSmartUnfoldingDefAux___closed__2); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/WF/GuessLex.c b/stage0/stdlib/Lean/Elab/PreDefinition/WF/GuessLex.c index deb8496e4a93..5f10517fc8c0 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/WF/GuessLex.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/WF/GuessLex.c @@ -63,7 +63,6 @@ LEAN_EXPORT uint8_t l_Lean_Expr_hasAnyFVar_visit___at_Lean_Elab_WF_GuessLex_mayO LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_WF_GuessLex_explainMutualFailure___spec__9___boxed(lean_object**); static lean_object* l_Lean_Elab_WF_guessLex___closed__1; static lean_object* l_Lean_Elab_WF_GuessLex_collectRecCalls___lambda__5___closed__1; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_RecCallCache_prettyEntry(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_WF_GuessLex_explainMutualFailure___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -73,6 +72,7 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_exp LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__24(lean_object*); static lean_object* l_Lean_Elab_WF_GuessLex_filterSubsumed___lambda__2___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_collectHeaders___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_WF_GuessLex_GuessLexRel_toNatRel___closed__17; LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__32___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Elab_WF_GuessLex_mkProdElem___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -102,6 +102,7 @@ lean_object* l_Lean_Meta_isExprDefEq(lean_object*, lean_object*, lean_object*, l static lean_object* l___private_Lean_Elab_PreDefinition_WF_GuessLex_0__Lean_Elab_WF_GuessLex_reprGuessLexRel____x40_Lean_Elab_PreDefinition_WF_GuessLex___hyg_4223____closed__5; lean_object* l_Lean_FileMap_toPosition(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_getMatcherInfo_x3f___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__2___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_WF_GuessLex_RecCallWithContext_posString___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__25___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__26___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -137,7 +138,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_measureHeader(lean_object*, lea static lean_object* l_List_forIn_loop___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__14___rarg___closed__2; static lean_object* l_Lean_Elab_WF_GuessLex_withRecApps___rarg___closed__4; static lean_object* l___private_Lean_Elab_PreDefinition_WF_GuessLex_0__Lean_Elab_WF_GuessLex_reprGuessLexRel____x40_Lean_Elab_PreDefinition_WF_GuessLex___hyg_4223____closed__10; -uint8_t l_Array_contains___at_Lean_findField_x3f___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Elab_WF_GuessLex_filterSubsumed___spec__6___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_Std_Range_forIn_x27_loop___at_Lean_Elab_WF_GuessLex_naryVarNames___spec__1___closed__1; LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Elab_WF_GuessLex_solve_go___spec__2___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*); @@ -236,9 +236,9 @@ LEAN_EXPORT lean_object* l_Lean_Meta_lambdaBoundedTelescope___at_Lean_Elab_WF_Gu LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_withRecApps___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_MatcherApp_inferMatchType___spec__9(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_forInAux___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__6___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_forIn___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__5(lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_WF_GuessLex_0__Lean_Elab_WF_GuessLex_reprGuessLexRel____x40_Lean_Elab_PreDefinition_WF_GuessLex___hyg_4223____closed__25; LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Elab_WF_GuessLex_formatTable___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_WF_GuessLex_explainMutualFailure___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -296,7 +296,6 @@ lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_logAt___at_Lean_Elab_Term_reportUnsolvedGoals___spec__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_WF_GuessLex_GuessLexRel_toNatRel___closed__20; LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_withRecApps_containsRecFn(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_WF_GuessLex_collectRecCalls___lambda__2___closed__3; size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_explainMutualFailure___spec__12___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -324,6 +323,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_withRecApps_loop___rarg___lambd LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_formatTable(lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_WF_GuessLex_generateCombinations_x3f_go___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__10___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_WF_GuessLex_0__Lean_Elab_WF_GuessLex_reprGuessLexRel____x40_Lean_Elab_PreDefinition_WF_GuessLex___hyg_4223____boxed(lean_object*, lean_object*); uint8_t lean_expr_eqv(lean_object*, lean_object*); @@ -340,10 +340,10 @@ lean_object* lean_nat_to_int(lean_object*); lean_object* l_Lean_MessageData_ofSyntax(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_WF_GuessLex_generateMeasures___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_WF_GuessLex_collectRecCalls___lambda__3___closed__1; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_toTerminationArguments(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getConstInfo___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__3___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_WF_GuessLex_filterSubsumed___lambda__2___closed__4; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_WF_guessLex___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_solve_go___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__9(lean_object*, lean_object*); @@ -365,7 +365,6 @@ lean_object* l_Lean_Name_getPrefix(lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_WF_GuessLex_explainNonMutualFailure___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_WF_GuessLex_naryVarNames_freshen___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__25___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__1(uint8_t, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__18___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_WF_GuessLex_isNatCmp___closed__5; static lean_object* l_Lean_Elab_WF_GuessLex_collectRecCalls___lambda__2___closed__4; @@ -431,7 +430,6 @@ lean_object* lean_st_mk_ref(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__12___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_to_list(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_WF_guessLex___spec__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_WF_GuessLex_mayOmitSizeOf___closed__8; lean_object* l_Lean_Expr_appFnCleanup(lean_object*, lean_object*); @@ -451,6 +449,7 @@ static lean_object* l___private_Lean_Elab_PreDefinition_WF_GuessLex_0__Lean_Elab static lean_object* l_Lean_Elab_WF_GuessLex_GuessLexRel_toNatRel___closed__27; static lean_object* l_Lean_Elab_WF_guessLex___lambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_evalRecCall___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_WF_GuessLex_explainMutualFailure___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_complexMeasures___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__11___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -461,7 +460,6 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_guessLex___s extern lean_object* l_Lean_instInhabitedExpr; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__10___lambda__1(lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_withRecApps_processApp(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__1___rarg___lambda__3(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_WF_GuessLex_explainNonMutualFailure___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_isNatCmp(lean_object*); @@ -520,6 +518,7 @@ lean_object* l_Lean_LocalContext_setUserName(lean_object*, lean_object*, lean_ob LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Elab_WF_GuessLex_solve_go___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_WF_GuessLex_withRecApps___rarg___closed__7; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_WF_GuessLex_evalRecCall___spec__3___lambda__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_reportTermArgs___spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_saveState___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_WF_guessLex___spec__6(size_t, size_t, lean_object*); @@ -531,13 +530,12 @@ LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Elab_WF_GuessLex_s LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutErrToSorry___at_Lean_Elab_WF_GuessLex_evalRecCall___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_WF_GuessLex_mayOmitSizeOf___closed__6; LEAN_EXPORT lean_object* l_Lean_Expr_hasAnyFVar_visit___at_Lean_Elab_WF_GuessLex_mayOmitSizeOf___spec__1___boxed(lean_object*, lean_object*); -static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_withRecApps_containsRecFn___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__17___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Elab_WF_GuessLex_formatTable___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_WF_guessLex___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_WF_GuessLex_explainMutualFailure___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_WF_guessLex___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_WF_GuessLex_evalRecCall___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_instInhabitedMeasure; @@ -570,7 +568,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_showInferredTerminationBy; lean_object* l_Array_append___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_WF_GuessLex_explainMutualFailure___spec__8___boxed(lean_object**); LEAN_EXPORT uint8_t l_Lean_Elab_WF_GuessLex_GuessLexRel_ofNat(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Elab_WF_GuessLex_formatTable___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Elab_WF_GuessLex_evalRecCall___spec__3___lambda__8___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__31___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -600,7 +597,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_GuessLexRel_noConfusion(lean_ob LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_evalRecCall(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_WF_guessLex___lambda__1___closed__7; LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_solve_go___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Elab_WF_GuessLex_evalRecCall___spec__3___closed__4; static size_t l_Lean_Elab_WF_GuessLex_generateMeasures___closed__3; @@ -648,6 +644,7 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_com static lean_object* l_Lean_Elab_WF_GuessLex_withRecApps___rarg___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_WF_guessLex___spec__3___boxed(lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_WF_GuessLex_GuessLexRel_toNatRel___closed__2; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_withUserNames___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_getMatcherInfo_x3f___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -668,7 +665,7 @@ lean_object* l_Lean_Elab_Term_TermElabM_run___rarg(lean_object*, lean_object*, l LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_Measure_toString(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_WF_guessLex___spec__1(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__1___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_WF_GuessLex_GuessLexRel_toNatRel___closed__26; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_solve_go___spec__1___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_getLocalInstances(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -695,6 +692,7 @@ static lean_object* l_Lean_Elab_WF_GuessLex_filterSubsumed___lambda__2___closed_ LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_solve_go___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_solve_go___at_Lean_Elab_WF_guessLex___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_StateRefT_x27_lift(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isConstOf(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__8(lean_object*, lean_object*); lean_object* lean_array_set(lean_object*, lean_object*, lean_object*); @@ -706,7 +704,7 @@ static lean_object* l_Lean_Elab_WF_GuessLex_withRecApps___rarg___lambda__1___clo LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__8___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_forM___at_Lean_Elab_WF_GuessLex_evalRecCall___spec__1___closed__2; lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_SavedLocalContext_run___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_type(lean_object*); lean_object* l_Lean_isTracingEnabledFor___at_Lean_Elab_Tactic_evalTactic_handleEx___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -754,7 +752,6 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_WF_GuessLex_wi LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__10___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__25___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_WF_GuessLex_evalRecCall___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__12(lean_object*, lean_object*); static lean_object* l_Lean_Elab_WF_GuessLex_GuessLexRel_toNatRel___closed__15; LEAN_EXPORT lean_object* l_Array_isEqvAux___at_Lean_Elab_WF_GuessLex_filterSubsumed___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -770,6 +767,7 @@ static lean_object* l_Lean_Elab_WF_GuessLex_isNatCmp___closed__4; lean_object* l_Array_ofSubarray___rarg(lean_object*); LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__10___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_WF_GuessLex_explainFailure___closed__5; LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_explainMutualFailure(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -779,6 +777,8 @@ static lean_object* l___private_Lean_Elab_PreDefinition_WF_GuessLex_0__Lean_Elab LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__18___boxed(lean_object*, lean_object*); static lean_object* l_List_forM___at_Lean_Elab_WF_GuessLex_evalRecCall___spec__1___closed__1; static lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__21___rarg___lambda__2___closed__2; +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_withRecApps_processApp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_instDecidableEqGuessLexRel___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Elab_WF_GuessLex_filterSubsumed___spec__6(lean_object*); @@ -789,6 +789,7 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_WF_GuessLex_withRecApp static lean_object* l_Lean_Elab_WF_GuessLex_explainFailure___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_filterSubsumed___lambda__1___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_withRecApps_loop___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__1(uint8_t, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_lambdaBoundedTelescope___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__28(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_inspectCall(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_sub(size_t, size_t); @@ -860,7 +861,6 @@ uint8_t l_Lean_isAuxRecursorWithSuffix(lean_object*, lean_object*, lean_object*) lean_object* lean_array_get_size(lean_object*); LEAN_EXPORT lean_object* l_Lean_resolveGlobalName___at_Lean_Elab_WF_GuessLex_naryVarNames_freshen___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_evalRecCall___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__13(lean_object*, lean_object*); static lean_object* l_Lean_Elab_WF_GuessLex_evalRecCall___lambda__3___closed__1; LEAN_EXPORT uint8_t l_Lean_Elab_WF_GuessLex_instDecidableEqGuessLexRel(uint8_t, uint8_t); @@ -896,6 +896,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_SavedLocalContext_run(lean_obje static lean_object* l_Lean_Elab_WF_GuessLex_instInhabitedMeasure___closed__1; static lean_object* l_Lean_Elab_WF_GuessLex_RecCallWithContext_posString___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_solve___at_Lean_Elab_WF_guessLex___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__22(lean_object*, lean_object*); uint8_t l_Lean_Expr_isFVar(lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_WF_GuessLex_formatTable___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -928,7 +929,6 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_com LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_ReaderT_instMonad___rarg(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_explainMutualFailure___spec__12___closed__10; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__31(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_isEqvAux___at_Lean_Elab_WF_GuessLex_filterSubsumed___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__30___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1157,7 +1157,7 @@ if (x_9 == 0) lean_object* x_10; lean_object* x_11; uint8_t x_12; x_10 = lean_ctor_get(x_8, 0); x_11 = lean_ctor_get(x_8, 1); -x_12 = l_Array_contains___at_Lean_findField_x3f___spec__1(x_1, x_2); +x_12 = l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(x_1, x_2); if (x_12 == 0) { uint8_t x_13; @@ -1200,7 +1200,7 @@ x_21 = lean_ctor_get(x_8, 1); lean_inc(x_21); lean_inc(x_20); lean_dec(x_8); -x_22 = l_Array_contains___at_Lean_findField_x3f___spec__1(x_1, x_2); +x_22 = l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(x_1, x_2); if (x_22 == 0) { uint8_t x_23; @@ -3455,7 +3455,7 @@ return x_56; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__1(uint8_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__1(uint8_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; @@ -3506,7 +3506,7 @@ return x_21; } } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1() { _start: { lean_object* x_1; lean_object* x_2; @@ -3515,7 +3515,7 @@ x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; lean_object* x_17; size_t x_18; lean_object* x_19; size_t x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; @@ -3539,7 +3539,7 @@ x_22 = lean_box(x_4); x_23 = lean_box_usize(x_18); x_24 = lean_box_usize(x_20); lean_inc(x_14); -x_25 = lean_alloc_closure((void*)(l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__1___boxed), 12, 7); +x_25 = lean_alloc_closure((void*)(l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__1___boxed), 12, 7); lean_closure_set(x_25, 0, x_22); lean_closure_set(x_25, 1, x_5); lean_closure_set(x_25, 2, x_14); @@ -3550,7 +3550,7 @@ lean_closure_set(x_25, 6, x_21); if (x_16 == 0) { lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_26 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_27 = l_outOfBounds___rarg(x_26); x_28 = l_Lean_Elab_WF_GuessLex_withUserNames___rarg(x_14, x_27, x_25, x_7, x_8, x_9, x_10, x_11); lean_dec(x_14); @@ -3566,7 +3566,7 @@ return x_30; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { lean_object* x_15; uint8_t x_16; @@ -3586,7 +3586,7 @@ x_21 = lean_box(x_4); lean_inc(x_7); lean_inc(x_3); lean_inc(x_2); -x_22 = lean_alloc_closure((void*)(l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___boxed), 11, 4); +x_22 = lean_alloc_closure((void*)(l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___boxed), 11, 4); lean_closure_set(x_22, 0, x_2); lean_closure_set(x_22, 1, x_3); lean_closure_set(x_22, 2, x_7); @@ -3674,7 +3674,7 @@ x_10 = lean_unsigned_to_nat(1u); x_11 = lean_nat_dec_lt(x_10, x_9); x_12 = lean_mk_empty_array_with_capacity(x_9); x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2(x_1, x_2, x_3, x_11, x_1, x_9, x_13, lean_box(0), x_12, x_4, x_5, x_6, x_7, x_8); +x_14 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2(x_1, x_2, x_3, x_11, x_1, x_9, x_13, lean_box(0), x_12, x_4, x_5, x_6, x_7, x_8); return x_14; } } @@ -3718,7 +3718,7 @@ lean_dec(x_3); return x_16; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { uint8_t x_13; size_t x_14; size_t x_15; lean_object* x_16; @@ -3728,32 +3728,32 @@ x_14 = lean_unbox_usize(x_5); lean_dec(x_5); x_15 = lean_unbox_usize(x_6); lean_dec(x_6); -x_16 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__1(x_13, x_2, x_3, x_4, x_14, x_15, x_7, x_8, x_9, x_10, x_11, x_12); +x_16 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__1(x_13, x_2, x_3, x_4, x_14, x_15, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_4); lean_dec(x_3); return x_16; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { uint8_t x_12; lean_object* x_13; x_12 = lean_unbox(x_4); lean_dec(x_4); -x_13 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2(x_1, x_2, x_3, x_12, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_13 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2(x_1, x_2, x_3, x_12, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_6); lean_dec(x_3); lean_dec(x_2); return x_13; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { uint8_t x_15; lean_object* x_16; x_15 = lean_unbox(x_4); lean_dec(x_4); -x_16 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2(x_1, x_2, x_3, x_15, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +x_16 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2(x_1, x_2, x_3, x_15, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); lean_dec(x_5); lean_dec(x_1); return x_16; @@ -18292,7 +18292,7 @@ lean_closure_set(x_27, 6, x_1); if (x_24 == 0) { lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_28 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_28 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_29 = l_outOfBounds___rarg(x_28); x_30 = lean_alloc_closure((void*)(l_Lean_Elab_WF_GuessLex_withUserNames___rarg___boxed), 8, 3); lean_closure_set(x_30, 0, x_22); @@ -18466,140 +18466,140 @@ return x_24; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, size_t x_6, size_t x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -uint8_t x_14; -x_14 = lean_usize_dec_lt(x_7, x_6); -if (x_14 == 0) +uint8_t x_13; +x_13 = lean_usize_dec_lt(x_6, x_5); +if (x_13 == 0) { -lean_object* x_15; -lean_dec(x_12); +lean_object* x_14; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_2); -x_15 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_15, 0, x_8); -lean_ctor_set(x_15, 1, x_13); -return x_15; +lean_dec(x_8); +lean_dec(x_1); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_7); +lean_ctor_set(x_14, 1, x_12); +return x_14; } else { -lean_object* x_16; lean_object* x_17; uint8_t x_18; -x_16 = lean_array_uget(x_5, x_7); -x_17 = lean_ctor_get(x_16, 1); -lean_inc(x_17); -x_18 = lean_nat_dec_eq(x_17, x_4); -lean_dec(x_17); -if (x_18 == 0) -{ -size_t x_19; size_t x_20; +lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_15 = lean_array_uget(x_4, x_6); +x_16 = lean_ctor_get(x_15, 1); +lean_inc(x_16); +x_17 = lean_nat_dec_eq(x_16, x_3); lean_dec(x_16); -x_19 = 1; -x_20 = lean_usize_add(x_7, x_19); -x_7 = x_20; +if (x_17 == 0) +{ +size_t x_18; size_t x_19; +lean_dec(x_15); +x_18 = 1; +x_19 = lean_usize_add(x_6, x_18); +x_6 = x_19; goto _start; } else { -lean_object* x_22; lean_object* x_23; -x_22 = lean_box(0); -lean_inc(x_12); +lean_object* x_21; lean_object* x_22; +x_21 = lean_box(0); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_2); -x_23 = l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__10___lambda__4(x_16, x_2, x_3, x_4, x_8, x_22, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_23) == 0) +lean_inc(x_8); +lean_inc(x_1); +x_22 = l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__10___lambda__4(x_15, x_1, x_2, x_3, x_7, x_21, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_22) == 0) { -lean_object* x_24; -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -if (lean_obj_tag(x_24) == 0) +lean_object* x_23; +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +if (lean_obj_tag(x_23) == 0) { -uint8_t x_25; -lean_dec(x_12); +uint8_t x_24; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_2); -x_25 = !lean_is_exclusive(x_23); -if (x_25 == 0) +lean_dec(x_8); +lean_dec(x_1); +x_24 = !lean_is_exclusive(x_22); +if (x_24 == 0) { -lean_object* x_26; lean_object* x_27; +lean_object* x_25; lean_object* x_26; +x_25 = lean_ctor_get(x_22, 0); +lean_dec(x_25); x_26 = lean_ctor_get(x_23, 0); -lean_dec(x_26); -x_27 = lean_ctor_get(x_24, 0); -lean_inc(x_27); -lean_dec(x_24); -lean_ctor_set(x_23, 0, x_27); -return x_23; +lean_inc(x_26); +lean_dec(x_23); +lean_ctor_set(x_22, 0, x_26); +return x_22; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_28 = lean_ctor_get(x_23, 1); +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_22, 1); +lean_inc(x_27); +lean_dec(x_22); +x_28 = lean_ctor_get(x_23, 0); lean_inc(x_28); lean_dec(x_23); -x_29 = lean_ctor_get(x_24, 0); -lean_inc(x_29); -lean_dec(x_24); -x_30 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_30, 0, x_29); -lean_ctor_set(x_30, 1, x_28); -return x_30; +x_29 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_27); +return x_29; } } else { -lean_object* x_31; lean_object* x_32; size_t x_33; size_t x_34; -x_31 = lean_ctor_get(x_23, 1); +lean_object* x_30; lean_object* x_31; size_t x_32; size_t x_33; +x_30 = lean_ctor_get(x_22, 1); +lean_inc(x_30); +lean_dec(x_22); +x_31 = lean_ctor_get(x_23, 0); lean_inc(x_31); lean_dec(x_23); -x_32 = lean_ctor_get(x_24, 0); -lean_inc(x_32); -lean_dec(x_24); -x_33 = 1; -x_34 = lean_usize_add(x_7, x_33); -x_7 = x_34; -x_8 = x_32; -x_13 = x_31; +x_32 = 1; +x_33 = lean_usize_add(x_6, x_32); +x_6 = x_33; +x_7 = x_31; +x_12 = x_30; goto _start; } } else { -uint8_t x_36; -lean_dec(x_12); +uint8_t x_35; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_2); -x_36 = !lean_is_exclusive(x_23); -if (x_36 == 0) +lean_dec(x_8); +lean_dec(x_1); +x_35 = !lean_is_exclusive(x_22); +if (x_35 == 0) { -return x_23; +return x_22; } else { -lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_37 = lean_ctor_get(x_23, 0); -x_38 = lean_ctor_get(x_23, 1); -lean_inc(x_38); +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_22, 0); +x_37 = lean_ctor_get(x_22, 1); lean_inc(x_37); -lean_dec(x_23); -x_39 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_39, 0, x_37); -lean_ctor_set(x_39, 1, x_38); -return x_39; +lean_inc(x_36); +lean_dec(x_22); +x_38 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_38, 0, x_36); +lean_ctor_set(x_38, 1, x_37); +return x_38; } } } } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__11(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__11(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { lean_object* x_15; uint8_t x_16; @@ -18619,7 +18619,7 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_2); -x_22 = l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__10(x_1, x_2, x_3, x_7, x_4, x_19, x_20, x_21, x_10, x_11, x_12, x_13, x_14); +x_22 = l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__10(x_2, x_3, x_7, x_4, x_19, x_20, x_21, x_10, x_11, x_12, x_13, x_14); if (lean_obj_tag(x_22) == 0) { lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; @@ -18693,7 +18693,7 @@ lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; x_10 = lean_array_get_size(x_1); x_11 = lean_mk_empty_array_with_capacity(x_10); x_12 = lean_unsigned_to_nat(0u); -x_13 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__11(x_1, x_2, x_3, x_4, x_1, x_10, x_12, lean_box(0), x_11, x_5, x_6, x_7, x_8, x_9); +x_13 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__11(x_1, x_2, x_3, x_4, x_1, x_10, x_12, lean_box(0), x_11, x_5, x_6, x_7, x_8, x_9); return x_13; } } @@ -18920,27 +18920,26 @@ lean_dec(x_3); return x_12; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -size_t x_14; size_t x_15; lean_object* x_16; +size_t x_13; size_t x_14; lean_object* x_15; +x_13 = lean_unbox_usize(x_5); +lean_dec(x_5); x_14 = lean_unbox_usize(x_6); lean_dec(x_6); -x_15 = lean_unbox_usize(x_7); -lean_dec(x_7); -x_16 = l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__10(x_1, x_2, x_3, x_4, x_5, x_14, x_15, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_5); +x_15 = l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__10(x_1, x_2, x_3, x_4, x_13, x_14, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_1); -return x_16; +lean_dec(x_2); +return x_15; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { lean_object* x_15; -x_15 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__11(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +x_15 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__11(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); @@ -22629,7 +22628,7 @@ if (x_10 == 0) { lean_object* x_50; lean_object* x_51; lean_dec(x_6); -x_50 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_50 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_51 = l_outOfBounds___rarg(x_50); x_14 = x_51; goto block_49; @@ -22650,7 +22649,7 @@ if (x_12 == 0) { lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_dec(x_11); -x_16 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_16 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_17 = l_outOfBounds___rarg(x_16); x_18 = lean_array_get_size(x_17); x_19 = lean_mk_array(x_18, x_5); @@ -22828,7 +22827,7 @@ if (x_50 == 0) { lean_object* x_51; lean_object* x_52; lean_object* x_53; uint8_t x_54; lean_dec(x_12); -x_51 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_51 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_52 = l_outOfBounds___rarg(x_51); x_53 = lean_array_get_size(x_52); x_54 = lean_nat_dec_lt(x_3, x_53); @@ -23094,7 +23093,7 @@ if (x_106 == 0) { lean_object* x_107; lean_object* x_108; lean_object* x_109; uint8_t x_110; lean_dec(x_70); -x_107 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_107 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_108 = l_outOfBounds___rarg(x_107); x_109 = lean_array_get_size(x_108); x_110 = lean_nat_dec_lt(x_3, x_109); @@ -23392,7 +23391,7 @@ if (x_46 == 0) { lean_object* x_47; lean_object* x_48; lean_dec(x_11); -x_47 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_47 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_48 = l_outOfBounds___rarg(x_47); x_15 = x_48; goto block_44; @@ -25867,7 +25866,7 @@ lean_ctor_set(x_7, 2, x_6); if (x_4 == 0) { lean_object* x_15; lean_object* x_16; -x_15 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_15 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_16 = l_outOfBounds___rarg(x_15); x_8 = x_16; goto block_14; @@ -28549,7 +28548,7 @@ lean_ctor_set(x_51, 1, x_29); if (x_32 == 0) { lean_object* x_167; lean_object* x_168; -x_167 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_167 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_168 = l_outOfBounds___rarg(x_167); x_52 = x_168; goto block_166; @@ -28579,7 +28578,7 @@ x_58 = lean_nat_dec_lt(x_18, x_57); if (x_58 == 0) { lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_59 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_59 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_60 = l_outOfBounds___rarg(x_59); x_61 = lean_array_get_size(x_60); lean_dec(x_60); @@ -28693,7 +28692,7 @@ lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean x_85 = lean_array_fget(x_2, x_18); x_86 = lean_array_get_size(x_85); lean_dec(x_85); -x_87 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_87 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_88 = lean_unsigned_to_nat(0u); x_89 = lean_unsigned_to_nat(1u); lean_inc(x_86); @@ -28811,7 +28810,7 @@ if (x_112 == 0) { lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_dec(x_17); -x_113 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_113 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_114 = l_outOfBounds___rarg(x_113); x_115 = lean_array_get_size(x_114); lean_dec(x_114); @@ -29124,7 +29123,7 @@ lean_ctor_set(x_209, 1, x_187); if (x_190 == 0) { lean_object* x_317; lean_object* x_318; -x_317 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_317 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_318 = l_outOfBounds___rarg(x_317); x_210 = x_318; goto block_316; @@ -29154,7 +29153,7 @@ x_216 = lean_nat_dec_lt(x_18, x_215); if (x_216 == 0) { lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; -x_217 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_217 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_218 = l_outOfBounds___rarg(x_217); x_219 = lean_array_get_size(x_218); lean_dec(x_218); @@ -29265,7 +29264,7 @@ lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; x_241 = lean_array_fget(x_2, x_18); x_242 = lean_array_get_size(x_241); lean_dec(x_241); -x_243 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_243 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_244 = lean_unsigned_to_nat(0u); x_245 = lean_unsigned_to_nat(1u); lean_inc(x_242); @@ -29380,7 +29379,7 @@ if (x_266 == 0) { lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_dec(x_17); -x_267 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_267 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_268 = l_outOfBounds___rarg(x_267); x_269 = lean_array_get_size(x_268); lean_dec(x_268); @@ -30232,7 +30231,7 @@ if (x_28 == 0) { lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_dec(x_2); -x_29 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_29 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_30 = l_outOfBounds___rarg(x_29); x_31 = l_Lean_Elab_WF_GuessLex_explainNonMutualFailure(x_30, x_3, x_4, x_5, x_6, x_7, x_8); if (lean_obj_tag(x_31) == 0) @@ -30874,7 +30873,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; @@ -30986,7 +30985,7 @@ return x_31; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; size_t x_19; size_t x_20; lean_object* x_21; lean_object* x_22; @@ -31002,7 +31001,7 @@ x_19 = lean_array_size(x_4); x_20 = 0; lean_inc(x_7); x_21 = l_Array_mapMUnsafe_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__1(x_3, x_5, x_7, x_19, x_20, x_4); -x_22 = lean_alloc_closure((void*)(l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2___lambda__1), 7, 2); +x_22 = lean_alloc_closure((void*)(l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2___lambda__1), 7, 2); lean_closure_set(x_22, 0, x_21); lean_closure_set(x_22, 1, x_7); if (x_18 == 0) @@ -31024,7 +31023,7 @@ return x_26; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { lean_object* x_16; uint8_t x_17; @@ -31046,7 +31045,7 @@ lean_dec(x_20); if (x_22 == 0) { lean_object* x_39; lean_object* x_40; -x_39 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_39 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_40 = l_outOfBounds___rarg(x_39); x_24 = x_40; goto block_38; @@ -31061,12 +31060,12 @@ goto block_38; block_38: { lean_object* x_25; lean_object* x_26; uint8_t x_27; lean_object* x_28; -x_25 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_25 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; lean_inc(x_5); lean_inc(x_8); lean_inc(x_3); lean_inc(x_2); -x_26 = lean_alloc_closure((void*)(l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2___lambda__2___boxed), 13, 6); +x_26 = lean_alloc_closure((void*)(l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2___lambda__2___boxed), 13, 6); lean_closure_set(x_26, 0, x_2); lean_closure_set(x_26, 1, x_3); lean_closure_set(x_26, 2, x_8); @@ -31157,7 +31156,7 @@ lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; x_11 = lean_array_get_size(x_1); x_12 = lean_mk_empty_array_with_capacity(x_11); x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2(x_1, x_2, x_3, x_4, x_5, x_1, x_11, x_13, lean_box(0), x_12, x_6, x_7, x_8, x_9, x_10); +x_14 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2(x_1, x_2, x_3, x_4, x_5, x_1, x_11, x_13, lean_box(0), x_12, x_6, x_7, x_8, x_9, x_10); return x_14; } } @@ -31175,11 +31174,11 @@ lean_dec(x_1); return x_9; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { lean_object* x_14; -x_14 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +x_14 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); lean_dec(x_8); lean_dec(x_5); lean_dec(x_3); @@ -31187,11 +31186,11 @@ lean_dec(x_2); return x_14; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { lean_object* x_16; -x_16 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +x_16 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); lean_dec(x_6); lean_dec(x_4); lean_dec(x_1); @@ -35204,8 +35203,8 @@ l_Subarray_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__1_ lean_mark_persistent(l_Subarray_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__1___closed__1); l_Subarray_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__1___closed__2 = _init_l_Subarray_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__1___closed__2(); lean_mark_persistent(l_Subarray_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__1___closed__2); -l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1 = _init_l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1); +l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1 = _init_l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1); l_Lean_Elab_WF_GuessLex_withRecApps_processRec___rarg___closed__1 = _init_l_Lean_Elab_WF_GuessLex_withRecApps_processRec___rarg___closed__1(); lean_mark_persistent(l_Lean_Elab_WF_GuessLex_withRecApps_processRec___rarg___closed__1); l_Lean_getConstInfo___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__3___rarg___closed__1 = _init_l_Lean_getConstInfo___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__3___rarg___closed__1(); diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/WF/Main.c b/stage0/stdlib/Lean/Elab/PreDefinition/WF/Main.c index 30022192c2b0..4f5f5d88f089 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/WF/Main.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/WF/Main.c @@ -7087,7 +7087,7 @@ lean_dec(x_33); x_35 = lean_ctor_get(x_15, 2); lean_inc(x_35); lean_dec(x_15); -x_36 = lean_ctor_get(x_35, 1); +x_36 = lean_ctor_get(x_35, 2); lean_inc(x_36); lean_dec(x_35); x_37 = lean_array_get_size(x_36); @@ -7244,7 +7244,7 @@ lean_dec(x_66); x_68 = lean_ctor_get(x_15, 2); lean_inc(x_68); lean_dec(x_15); -x_69 = lean_ctor_get(x_68, 1); +x_69 = lean_ctor_get(x_68, 2); lean_inc(x_69); lean_dec(x_68); x_70 = lean_array_get_size(x_69); diff --git a/stage0/stdlib/Lean/Elab/Print.c b/stage0/stdlib/Lean/Elab/Print.c index aa19353fb761..f56889072258 100644 --- a/stage0/stdlib/Lean/Elab/Print.c +++ b/stage0/stdlib/Lean/Elab/Print.c @@ -31,6 +31,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_printI lean_object* lean_private_to_user_name(lean_object*); 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___private_Lean_Elab_Command_0__Lean_Elab_Command_elabCommandUsing___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_ConstantInfo_type(lean_object*); static lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_printStructure___closed__1; lean_object* l_Lean_ConstantInfo_levelParams(lean_object*); @@ -61,6 +62,7 @@ static lean_object* l___regBuiltin_Lean_Elab_Command_elabPrintEqns_declRange__1_ static lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_mkHeader___closed__6; static lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_printEqnsOf___closed__1; lean_object* lean_environment_find(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__1___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabPrintEqns_declRange__1___closed__4; lean_object* l_Lean_addBuiltinDeclarationRanges(lean_object*, lean_object*, lean_object*); @@ -94,14 +96,16 @@ static lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_printIdCore uint8_t lean_get_reducibility_status(lean_object*, lean_object*); uint8_t l_Lean_TagDeclarationExtension_isTagged(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forM___at_Lean_Elab_Command_elabPrintAxioms___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printStructure_doFields___spec__3___closed__3; static lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_mkHeader___closed__18; -lean_object* l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_printStructure_doFields(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescope___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printStructure_doFields___spec__4(lean_object*); static lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_printAxiomsOf___closed__4; extern lean_object* l_Lean_Elab_Command_commandElabAttribute; static lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_mkHeader___closed__13; +static lean_object* l_Lean_getConstInfo___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__1___closed__1; static lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_mkHeader___closed__24; static lean_object* l___regBuiltin_Lean_Elab_Command_elabPrint_declRange__1___closed__3; static lean_object* l_panic___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printIdCore___spec__1___closed__1; @@ -121,6 +125,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabPrintEqns_declRang LEAN_EXPORT lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_printDefLike___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_Print_0__Lean_Elab_Command_printStructure_doFields___spec__3___closed__2; lean_object* l_Lean_MessageData_ofFormat(lean_object*); +lean_object* l_Lean_Elab_getBetterRef(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabPrintAxioms__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabPrintAxioms___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_getEqnsFor_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -150,6 +155,7 @@ static lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_levelParams static lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_printIdCore___closed__9; static lean_object* l___regBuiltin_Lean_Elab_Command_elabPrintEqns_declRange__1___closed__1; static lean_object* l_Array_qsort_sort___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printAxiomsOf___spec__2___closed__1; +lean_object* l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabPrint__1___closed__2; lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -177,6 +183,7 @@ static lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_printAxioms lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallTelescopeReducingAuxAux___rarg(uint8_t, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescope___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printStructure_doFields___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_EXPORT lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_printStructure_doFields___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_getConstInfo___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__1___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Command_elabPrint_declRange__1___closed__1; static lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_printIdCore___closed__3; static lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_mkHeader___closed__1; @@ -207,7 +214,6 @@ uint8_t lean_nat_dec_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_printId(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabPrint___closed__10; LEAN_EXPORT lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_printStructure_doFields___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabPrintAxioms_declRange__1___closed__2; static lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_levelParamsToMessageData___closed__7; LEAN_EXPORT lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_printEqnsOf___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -257,6 +263,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabPrintEqns__1(lean_ static lean_object* l_List_forIn_loop___at___private_Lean_Elab_Print_0__Lean_Elab_Command_levelParamsToMessageData___spec__1___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_printEqnsOf(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forM___at_Lean_Elab_Command_elabPrintAxioms___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_collectAxioms___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printAxiomsOf___spec__1___closed__2; LEAN_EXPORT lean_object* l_Lean_getReducibilityStatus___at___private_Lean_Elab_Print_0__Lean_Elab_Command_mkHeader___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_uget(lean_object*, size_t); @@ -264,8 +271,8 @@ size_t lean_array_size(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_mkHeader_x27(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabPrint___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_printDefLike(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_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_Elab_Print_0__Lean_Elab_Command_printStructure_doFields___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_Print_0__Lean_Elab_Command_printIdCore___closed__6; static lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___closed__6; @@ -295,6 +302,7 @@ lean_object* l___private_Init_Data_Repr_0__Nat_reprFast(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_panic___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printStructure_doFields___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printStructure_doFields___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_throwError___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_printIdCore(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_mkHeader(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_printStructure___closed__8; @@ -1601,7 +1609,204 @@ lean_dec(x_5); return x_7; } } -LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___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_throwError___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___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; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_5 = l_Lean_Elab_Command_getRef(x_2, x_3, x_4); +x_6 = lean_ctor_get(x_5, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_5, 1); +lean_inc(x_7); +lean_dec(x_5); +x_8 = lean_ctor_get(x_2, 4); +lean_inc(x_8); +lean_inc(x_8); +x_9 = l_Lean_Elab_getBetterRef(x_6, x_8); +lean_dec(x_6); +x_10 = l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1(x_1, x_2, x_3, x_7); +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_12 = lean_ctor_get(x_10, 0); +x_13 = lean_ctor_get(x_10, 1); +x_14 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_12, x_8, x_2, x_3, x_13); +lean_dec(x_2); +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 0) +{ +lean_object* x_16; +x_16 = lean_ctor_get(x_14, 0); +lean_ctor_set(x_10, 1, x_16); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set_tag(x_14, 1); +lean_ctor_set(x_14, 0, x_10); +return x_14; +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_14, 0); +x_18 = lean_ctor_get(x_14, 1); +lean_inc(x_18); +lean_inc(x_17); +lean_dec(x_14); +lean_ctor_set(x_10, 1, x_17); +lean_ctor_set(x_10, 0, x_9); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_10); +lean_ctor_set(x_19, 1, 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; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_20 = lean_ctor_get(x_10, 0); +x_21 = lean_ctor_get(x_10, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_10); +x_22 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_20, x_8, x_2, x_3, x_21); +lean_dec(x_2); +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +if (lean_is_exclusive(x_22)) { + lean_ctor_release(x_22, 0); + lean_ctor_release(x_22, 1); + x_25 = x_22; +} else { + lean_dec_ref(x_22); + x_25 = lean_box(0); +} +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_9); +lean_ctor_set(x_26, 1, x_23); +if (lean_is_scalar(x_25)) { + x_27 = lean_alloc_ctor(1, 2, 0); +} else { + x_27 = x_25; + lean_ctor_set_tag(x_27, 1); +} +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_24); +return x_27; +} +} +} +static lean_object* _init_l_Lean_getConstInfo___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("unknown constant '", 18, 18); +return x_1; +} +} +static lean_object* _init_l_Lean_getConstInfo___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_getConstInfo___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__1___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__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_3, x_4); +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; +x_7 = lean_ctor_get(x_5, 0); +x_8 = lean_ctor_get(x_5, 1); +x_9 = lean_ctor_get(x_7, 0); +lean_inc(x_9); +lean_dec(x_7); +lean_inc(x_1); +x_10 = lean_environment_find(x_9, x_1); +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; +lean_free_object(x_5); +x_11 = lean_box(0); +x_12 = l_Lean_Expr_const___override(x_1, x_11); +x_13 = l_Lean_MessageData_ofExpr(x_12); +x_14 = l_Lean_getConstInfo___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__1___closed__2; +x_15 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_13); +x_16 = l___private_Lean_Elab_Print_0__Lean_Elab_Command_throwUnknownId___closed__4; +x_17 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_17, 0, x_15); +lean_ctor_set(x_17, 1, x_16); +x_18 = l_Lean_throwError___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__2(x_17, x_2, x_3, x_8); +return x_18; +} +else +{ +lean_object* x_19; +lean_dec(x_2); +lean_dec(x_1); +x_19 = lean_ctor_get(x_10, 0); +lean_inc(x_19); +lean_dec(x_10); +lean_ctor_set(x_5, 0, x_19); +return x_5; +} +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_20 = lean_ctor_get(x_5, 0); +x_21 = lean_ctor_get(x_5, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_5); +x_22 = lean_ctor_get(x_20, 0); +lean_inc(x_22); +lean_dec(x_20); +lean_inc(x_1); +x_23 = lean_environment_find(x_22, x_1); +if (lean_obj_tag(x_23) == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_24 = lean_box(0); +x_25 = l_Lean_Expr_const___override(x_1, x_24); +x_26 = l_Lean_MessageData_ofExpr(x_25); +x_27 = l_Lean_getConstInfo___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__1___closed__2; +x_28 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_26); +x_29 = l___private_Lean_Elab_Print_0__Lean_Elab_Command_throwUnknownId___closed__4; +x_30 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +x_31 = l_Lean_throwError___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__2(x_30, x_2, x_3, x_21); +return x_31; +} +else +{ +lean_object* x_32; lean_object* x_33; +lean_dec(x_2); +lean_dec(x_1); +x_32 = lean_ctor_get(x_23, 0); +lean_inc(x_32); +lean_dec(x_23); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_21); +return x_33; +} +} +} +} +LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { if (lean_obj_tag(x_2) == 0) @@ -1625,7 +1830,7 @@ x_9 = lean_ctor_get(x_2, 0); x_10 = lean_ctor_get(x_2, 1); lean_inc(x_4); lean_inc(x_9); -x_11 = l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9(x_9, x_4, x_5, x_6); +x_11 = l_Lean_getConstInfo___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__1(x_9, x_4, x_5, x_6); if (lean_obj_tag(x_11) == 0) { lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; @@ -1696,7 +1901,7 @@ lean_inc(x_26); lean_dec(x_2); lean_inc(x_4); lean_inc(x_26); -x_28 = l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9(x_26, x_4, x_5, x_6); +x_28 = l_Lean_getConstInfo___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__1(x_26, x_4, x_5, x_6); 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; @@ -1856,7 +2061,7 @@ x_23 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_23, 0, x_21); lean_ctor_set(x_23, 1, x_22); lean_inc(x_7); -x_24 = l_List_forIn_loop___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__1(x_14, x_5, x_23, x_7, x_8, x_13); +x_24 = l_List_forIn_loop___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__3(x_14, x_5, x_23, x_7, x_8, x_13); if (lean_obj_tag(x_24) == 0) { lean_object* x_25; lean_object* x_26; uint8_t x_27; lean_object* x_28; @@ -1924,7 +2129,7 @@ x_45 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_45, 0, x_43); lean_ctor_set(x_45, 1, x_44); lean_inc(x_7); -x_46 = l_List_forIn_loop___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__1(x_35, x_5, x_45, x_7, x_8, x_34); +x_46 = l_List_forIn_loop___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__3(x_35, x_5, x_45, x_7, x_8, x_34); if (lean_obj_tag(x_46) == 0) { lean_object* x_47; lean_object* x_48; uint8_t x_49; lean_object* x_50; @@ -1965,11 +2170,29 @@ return x_54; } } } -LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___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___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___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___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__2(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___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_getConstInfo___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__1(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___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: { lean_object* x_7; -x_7 = l_List_forIn_loop___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__1(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_List_forIn_loop___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__3(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_5); return x_7; } @@ -3505,7 +3728,7 @@ lean_ctor_set(x_25, 0, x_23); lean_ctor_set(x_25, 1, x_24); lean_inc(x_9); lean_inc(x_5); -x_26 = l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9(x_5, x_9, x_10, x_15); +x_26 = l_Lean_getConstInfo___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__1(x_5, x_9, x_10, x_15); 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; @@ -3640,7 +3863,7 @@ lean_ctor_set(x_66, 0, x_64); lean_ctor_set(x_66, 1, x_65); lean_inc(x_9); lean_inc(x_5); -x_67 = l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9(x_5, x_9, x_10, x_55); +x_67 = l_Lean_getConstInfo___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__1(x_5, x_9, x_10, x_55); 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; @@ -5443,7 +5666,7 @@ lean_object* x_10; lean_object* x_11; x_10 = lean_array_uget(x_1, x_3); lean_inc(x_5); lean_inc(x_10); -x_11 = l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9(x_10, x_5, x_6, x_7); +x_11 = l_Lean_getConstInfo___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__1(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; lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; uint8_t x_19; @@ -6112,6 +6335,10 @@ l___private_Lean_Elab_Print_0__Lean_Elab_Command_printDefLike___closed__4 = _ini lean_mark_persistent(l___private_Lean_Elab_Print_0__Lean_Elab_Command_printDefLike___closed__4); l___private_Lean_Elab_Print_0__Lean_Elab_Command_printQuot___closed__1 = _init_l___private_Lean_Elab_Print_0__Lean_Elab_Command_printQuot___closed__1(); lean_mark_persistent(l___private_Lean_Elab_Print_0__Lean_Elab_Command_printQuot___closed__1); +l_Lean_getConstInfo___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__1___closed__1 = _init_l_Lean_getConstInfo___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__1___closed__1(); +lean_mark_persistent(l_Lean_getConstInfo___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__1___closed__1); +l_Lean_getConstInfo___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__1___closed__2 = _init_l_Lean_getConstInfo___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__1___closed__2(); +lean_mark_persistent(l_Lean_getConstInfo___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___spec__1___closed__2); l___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___closed__1 = _init_l___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___closed__1(); lean_mark_persistent(l___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___closed__1); l___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___closed__2 = _init_l___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___closed__2(); diff --git a/stage0/stdlib/Lean/Elab/Quotation.c b/stage0/stdlib/Lean/Elab/Quotation.c index e6ec4af0a445..4ba5934acf72 100644 --- a/stage0/stdlib/Lean/Elab/Quotation.c +++ b/stage0/stdlib/Lean/Elab/Quotation.c @@ -29,7 +29,6 @@ lean_object* l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(lean_object*, lean_obj LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___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*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_markRhss___closed__5; static lean_object* l_Lean_Elab_Term_Quotation___aux__Lean__Elab__Quotation______macroRules__Lean__Elab__Term__Quotation__commandElab__stx__quot____1___closed__36; -static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__5; static lean_object* l_List_mapM_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__4___closed__7; LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Term_Quotation_match__syntax_expand___spec__9___rarg(lean_object*); static lean_object* l_Lean_Elab_Term_Quotation_ArrayStxBuilder_mkNode___closed__19; @@ -37,13 +36,13 @@ static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_ LEAN_EXPORT lean_object* l_List_foldlM___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___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*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__9___closed__4; static lean_object* l_Lean_Elab_Term_Quotation___aux__Lean__Elab__Quotation______macroRules__Lean__Elab__Term__Quotation__commandElab__stx__quot____1___closed__2; +static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__1; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__2___closed__10; lean_object* l_Lean_Syntax_mkNameLit(lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__9___closed__9; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_Quotation_ArrayStxBuilder_mkNode___closed__2; static lean_object* l_Lean_Elab_Term_Quotation___aux__Lean__Elab__Quotation______macroRules__Lean__Elab__Term__Quotation__commandElab__stx__quot____1___closed__7; -static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__2; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__3___closed__32; LEAN_EXPORT lean_object* l_Lean_Elab_Term_Quotation_ArrayStxBuilder_push(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_Quotation_match__syntax_expand___spec__10___boxed(lean_object*, lean_object*, lean_object*); @@ -75,13 +74,12 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quota static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__9___closed__11; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__9___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Term_Quotation_match__syntax_expand___lambda__4(lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6422____closed__3; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_noOpMatchAdaptPats___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_Quotation_match__syntax_expand___lambda__1(lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6426____closed__3; static lean_object* l_Lean_Elab_Term_Quotation_mkTuple___closed__2; lean_object* l_Lean_Elab_Term_Quotation_getPatternsVars(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_Quotation_mkTuple___closed__5; -LEAN_EXPORT lean_object* l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6426_(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_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__3___closed__12; static lean_object* l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed__32; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___lambda__1___closed__20; @@ -94,7 +92,6 @@ static lean_object* l_Lean_Elab_Term_Quotation_ArrayStxBuilder_mkNode___closed__ lean_object* l_Lean_Syntax_getQuotContent(lean_object*); static lean_object* l_Lean_Elab_Term_Quotation___aux__Lean__Elab__Quotation______macroRules__Lean__Elab__Term__Quotation__commandElab__stx__quot____1___closed__18; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__48; -static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__15; static lean_object* l_Lean_Elab_Term_Quotation_getQuotKind___closed__15; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__28; static lean_object* l_List_foldlM___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__17___closed__2; @@ -102,6 +99,7 @@ uint8_t l_List_all___rarg(lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__54; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_markRhss___closed__6; LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_deduplicate___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_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__7; LEAN_EXPORT lean_object* l_Array_sequenceMap_loop___at_Lean_Elab_Term_Quotation_match__syntax_expand___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed__21; @@ -109,33 +107,31 @@ static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_ static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__11___closed__5; LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__19(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed__11; +LEAN_EXPORT lean_object* l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6422_(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_Quotation_mkSyntaxQuotation___closed__2; static lean_object* l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed__33; lean_object* l_Lean_Elab_Term_Quotation_getAntiquotKindSpec_x3f(lean_object*); 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_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6412____closed__1; static lean_object* l_Lean_Elab_Term_Quotation_ArrayStxBuilder_mkNode___closed__32; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__21(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_Quotation_ArrayStxBuilder_mkNode___closed__40; static lean_object* l_Lean_Elab_Term_Quotation_ArrayStxBuilder_mkNode___closed__72; LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__26; -LEAN_EXPORT lean_object* l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6433_(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__3; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___lambda__1___closed__25; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_floatOutAntiquotTerms___lambda__1___closed__7; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__23___closed__14; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___lambda__1___closed__38; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_floatOutAntiquotTerms___lambda__1___closed__8; LEAN_EXPORT lean_object* l_Lean_Elab_Term_Quotation_elabNoErrorIfUnused(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint64_t lean_uint64_of_nat(lean_object*); static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___lambda__1___closed__28; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__3___closed__7; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__14___closed__6; lean_object* l_Lean_Elab_Term_elabTerm(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__15(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__10; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__27___closed__3; LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__14___closed__2; @@ -144,6 +140,7 @@ size_t lean_uint64_to_usize(uint64_t); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__41; static lean_object* l_Lean_Elab_Term_Quotation___aux__Lean__Elab__Quotation______macroRules__Lean__Elab__Term__Quotation__commandElab__stx__quot____1___closed__48; static lean_object* l_Lean_Elab_Term_Quotation_commandElab__stx__quot_____closed__7; +static lean_object* l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6415____closed__1; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__30___closed__1; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___closed__4; uint8_t l_Lean_Syntax_isAntiquotSuffixSplice(lean_object*); @@ -156,6 +153,7 @@ lean_object* l_Lean_Syntax_getId(lean_object*); static lean_object* l_Lean_Elab_Term_Quotation_ArrayStxBuilder_push___closed__1; static lean_object* l_Lean_Elab_Term_Quotation___aux__Lean__Elab__Quotation______macroRules__Lean__Elab__Term__Quotation__commandElab__stx__quot____1___closed__55; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__23___closed__22; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6443_(lean_object*); static lean_object* l_List_forIn_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_compileStxMatch___spec__4___closed__6; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__3___closed__5; LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__28(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -186,18 +184,18 @@ lean_object* lean_mk_array(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_Quotation___aux__Lean__Elab__Quotation______macroRules__Lean__Elab__Term__Quotation__commandElab__stx__quot____1___closed__50; static lean_object* l_Lean_Elab_Term_Quotation_ArrayStxBuilder_mkNode___closed__42; uint8_t lean_usize_dec_eq(size_t, size_t); +static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6436____closed__1; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___lambda__1___closed__2; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__38; LEAN_EXPORT lean_object* l_Array_sequenceMap___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_deduplicate___spec__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__23___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__16___closed__4; +static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__7; lean_object* l_Lean_Syntax_getArgs(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__19___boxed(lean_object**); static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___lambda__1___closed__33; -LEAN_EXPORT lean_object* l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962_(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__19; LEAN_EXPORT uint8_t l_List_beq___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__5(lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__13; static lean_object* l_Lean_Elab_Term_Quotation_instQuotePreresolvedMkStr1__lean___closed__8; lean_object* l_Lean_replaceRef(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_Quotation_ArrayStxBuilder_mkNode___closed__43; @@ -214,19 +212,18 @@ static lean_object* l_Lean_Elab_Term_Quotation_getQuotKind___closed__9; LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_floatOutAntiquotTerms___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getPos_x3f(lean_object*, uint8_t); lean_object* lean_array_fget(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6429____closed__1; static lean_object* l_Lean_Elab_Term_Quotation___aux__Lean__Elab__Quotation______macroRules__Lean__Elab__Term__Quotation__commandElab__stx__quot____1___closed__41; static lean_object* l_Lean_Elab_Term_Quotation___aux__Lean__Elab__Quotation______macroRules__Lean__Elab__Term__Quotation__commandElab__stx__quot____1___closed__38; static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__12___closed__3; static lean_object* l_Lean_Elab_Term_Quotation_mkTuple___closed__8; LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_deduplicate___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_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__1; lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_compileStxMatch___closed__6; lean_object* l_Lean_Syntax_getTailPos_x3f(lean_object*, uint8_t); static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getSepStxFromSplice___closed__19; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__8___closed__7; lean_object* l_Lean_Syntax_getAntiquotTerm(lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__14; LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__27(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___lambda__1___closed__11; static lean_object* l_Lean_Elab_Term_Quotation___aux__Lean__Elab__Quotation______macroRules__Lean__Elab__Term__Quotation__commandElab__stx__quot____1___closed__33; @@ -241,9 +238,9 @@ LEAN_EXPORT uint8_t l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_ static lean_object* l_Lean_Elab_Term_Quotation_instQuotePreresolvedMkStr1__lean___closed__7; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__14___closed__4; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_floatOutAntiquotTerms___lambda__1___closed__1; -static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6433____closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabNoErrorIfUnused__1(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23(lean_object*, lean_object*, size_t, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__13; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__27___closed__5; LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_quoteList___at_Lean_Elab_Term_Quotation_instQuotePreresolvedMkStr1__lean___spec__1(lean_object*); static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__25___closed__1; @@ -254,6 +251,7 @@ lean_object* l_Lean_addBuiltinDeclarationRanges(lean_object*, lean_object*, lean static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__10___closed__3; LEAN_EXPORT lean_object* l_Lean_resolveNamespaceCore___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__26___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed__12; +static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6436____closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___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_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__34; static lean_object* l_Lean_Elab_Term_Quotation___aux__Lean__Elab__Quotation______macroRules__Lean__Elab__Term__Quotation__commandElab__stx__quot____1___closed__5; @@ -293,7 +291,6 @@ static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_ static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getSepFromSplice___closed__1; static lean_object* l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed__26; lean_object* l_Lean_stringToMessageData(lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__10; LEAN_EXPORT lean_object* l_Lean_Elab_Term_Quotation_ArrayStxBuilder_mkNode___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_Quotation_commandElab__stx__quot_____closed__8; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -340,23 +337,26 @@ static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_ static lean_object* l_Lean_Elab_Term_Quotation_ArrayStxBuilder_mkNode___closed__24; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___lambda__1___closed__32; static lean_object* l_Lean_Elab_Term_Quotation_ArrayStxBuilder_mkNode___closed__23; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__68; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Term_Quotation_match__syntax_expand___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_string_utf8_byte_size(lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__14; +static lean_object* l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__9; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__23___closed__17; -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6433_(lean_object*); static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__23___closed__15; static lean_object* l_List_forIn_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_compileStxMatch___spec__4___closed__4; static lean_object* l___private_Init_Meta_0__Lean_quoteList___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__29___closed__5; static lean_object* l_Lean_Elab_Term_Quotation_mkTuple___closed__9; +static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6443____closed__2; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___lambda__1___closed__10; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__16___closed__7; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__21___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed__30; static lean_object* l_List_foldlM___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__17___closed__5; +static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__8; lean_object* l_Lean_Syntax_getNumArgs(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_compileStxMatch___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_Quotation_instReprMatchResult___closed__2; -static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__9; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__42; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_compileStxMatch___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_Lean_Elab_Term_Quotation_mkSyntaxQuotation(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -373,10 +373,12 @@ static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_ static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__40; LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo(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_resolveSectionVariable_loop___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__4; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getSepStxFromSplice___closed__7; LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__30___closed__2; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__10; +static lean_object* l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__5; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_compileStxMatch___closed__1; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___lambda__1___closed__4; LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___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*); @@ -387,7 +389,6 @@ static lean_object* l_Lean_Elab_Term_Quotation_ArrayStxBuilder_mkNode___closed__ LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_Quotation_ArrayStxBuilder_mkNode___closed__18; lean_object* l_List_appendTR___rarg(lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6440____closed__3; LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___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_Term_Quotation_mkSyntaxQuotation___closed__27; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__10___closed__16; @@ -397,18 +398,19 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_Quotation_addNamedQuotInfo(lean_object static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_compileStxMatch___spec__9(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_sequenceMap___at_Lean_Elab_Term_Quotation_match__syntax_expand___spec__1___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6436_(lean_object*); static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_floatOutAntiquotTerms___lambda__1___closed__14; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_markRhss___spec__4(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_Quotation_instReprMatchResult(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_Quotation_match__syntax_expand___lambda__4___closed__2; static lean_object* l_Lean_Elab_Term_Quotation_ArrayStxBuilder_empty___closed__1; -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6426_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968_(lean_object*); static lean_object* l_Lean_Elab_Term_Quotation_ArrayStxBuilder_mkNode___closed__71; static lean_object* l_Lean_Elab_Term_Quotation_getQuotKind___closed__19; -static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6433____closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Term_Quotation_stxQuot_expand(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_Quotation_ArrayStxBuilder_mkNode___closed__11; static lean_object* l_Lean_Elab_Term_Quotation_ArrayStxBuilder_mkNode___closed__10; +static lean_object* l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Term_Quotation_match__syntax_expand___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_foldrMUnsafe_fold___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__4___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_compileStxMatch___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*); @@ -419,6 +421,7 @@ LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Quotation_0__ static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___lambda__1___closed__37; static lean_object* l_Lean_Elab_Term_Quotation_instQuotePreresolvedMkStr1__lean___closed__17; static lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__1___rarg___closed__1; +static lean_object* l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__8; LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_Term_Quotation_getQuotKind___spec__2(lean_object*); static lean_object* l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed__40; @@ -440,7 +443,6 @@ static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_ static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__51; LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__18(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_checkUnusedAlts___spec__1___boxed(lean_object**); -static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6419____closed__1; static lean_object* l_Lean_Elab_Term_Quotation___aux__Lean__Elab__Quotation______macroRules__Lean__Elab__Term__Quotation__commandElab__stx__quot____1___closed__31; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_markRhss___spec__6___lambda__1___closed__2; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__25___closed__11; @@ -455,7 +457,6 @@ static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_ static lean_object* l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed__34; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___lambda__1___closed__13; static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabNoErrorIfUnused_declRange__1___closed__3; -static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6440____closed__1; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___lambda__1___closed__35; static lean_object* l_Lean_Elab_Term_Quotation_ArrayStxBuilder_mkNode___closed__22; LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_floatOutAntiquotTerms___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -525,21 +526,20 @@ lean_object* l_Lean_MessageData_ofFormat(lean_object*); lean_object* l_ReaderT_instMonadLift(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_noOpMatchAdaptPats(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed__22; -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6440_(lean_object*); lean_object* l_Lean_Elab_Term_Quotation_getAntiquotationIds(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkCIdentFrom(lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_quoteArray_go___at_Lean_Elab_Term_Quotation_ArrayStxBuilder_build___spec__3___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___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_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_getBetterRef(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__15; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_compileStxMatch___lambda__5___closed__7; -static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__1; +static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6422____closed__1; +static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__2; static lean_object* l_Lean_Elab_Term_Quotation_commandElab__stx__quot_____closed__12; LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__27(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__6; static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabNoErrorIfUnused__1___closed__1; static lean_object* l_Lean_Elab_Term_Quotation_instReprMatchResult___closed__8; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__14___closed__1; -static lean_object* l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__5; lean_object* l_outOfBounds___rarg(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___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_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_deduplicate___lambda__3___boxed(lean_object*, lean_object*); @@ -550,8 +550,8 @@ static lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Elab_Quotatio LEAN_EXPORT lean_object* l_Lean_Elab_Term_Quotation___aux__Lean__Elab__Quotation______macroRules__Lean__Elab__Term__Quotation__commandElab__stx__quot____1(lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__37; static lean_object* l_Lean_Elab_Term_Quotation_instReprMatchResult___closed__5; -static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__8; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__23___closed__7; +static lean_object* l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__4; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___lambda__1___closed__23; static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__3___closed__1; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__23___closed__19; @@ -562,6 +562,7 @@ static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_Quotation_match__syntax_expand___spec__7(size_t, size_t, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_Quotation_commandElab__stx__quot_____closed__9; +LEAN_EXPORT lean_object* l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6443_(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_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__8___closed__6; static lean_object* l_Lean_Elab_Term_Quotation_commandElab__stx__quot_____closed__2; 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*); @@ -616,6 +617,7 @@ static lean_object* l_Array_foldrMUnsafe_fold___at___private_Lean_Elab_Quotation static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__2___closed__6; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_Quotation_match__syntax_expand___spec__5(size_t, size_t, lean_object*); static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__8___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6429_(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__12; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_compileStxMatch___spec__6(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_Quotation_mkTuple___closed__7; @@ -663,7 +665,8 @@ static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_ static lean_object* l_Lean_Elab_Term_Quotation_commandElab__stx__quot_____closed__6; static lean_object* l_Lean_Elab_Term_Quotation_ArrayStxBuilder_mkNode___closed__73; lean_object* l_Lean_addMacroScope(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__9; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__69; +LEAN_EXPORT lean_object* l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6429_(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_Quotation_0__Lean_Elab_Term_Quotation_findUsedAlts_go___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* l_Lean_Core_withFreshMacroScope___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_floatOutAntiquotTerms___lambda__1___closed__12; @@ -711,12 +714,13 @@ static lean_object* l_Lean_Elab_Term_Quotation___aux__Lean__Elab__Quotation_____ lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__12(lean_object*, size_t, size_t, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__56; +static lean_object* l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__10; uint8_t l_Lean_Syntax_matchesNull(lean_object*, lean_object*); static lean_object* l___private_Init_Meta_0__Lean_quoteList___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__29___closed__3; uint8_t l_Lean_Syntax_isTokenAntiquot(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6412_(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_Quotation___aux__Lean__Elab__Quotation______macroRules__Lean__Elab__Term__Quotation__commandElab__stx__quot____1___closed__4; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__13; +static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__12; uint8_t l_Lean_Syntax_isIdent(lean_object*); LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_compileStxMatch___spec__5___lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_checkUnusedAlts___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -725,6 +729,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quota static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__14___closed__15; static lean_object* l_panic___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_compileStxMatch___spec__1___closed__1; static lean_object* l_Lean_Elab_Term_Quotation_instReprMatchResult___closed__14; +static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__16; static lean_object* l_Lean_Elab_Term_Quotation_instQuotePreresolvedMkStr1__lean___closed__15; lean_object* l_Lean_resolveGlobalName___at_Lean_Elab_Term_resolveLocalName_loop___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabMatchSyntax__1___closed__2; @@ -739,6 +744,7 @@ LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_Quotation_ma static lean_object* l_Lean_Elab_Term_Quotation_mkTuple___closed__14; lean_object* l_Array_eraseIdx___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldlM___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___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*); +static lean_object* l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__2; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___lambda__2___closed__3; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___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_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__67; @@ -756,15 +762,16 @@ static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Quotation_0_ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed__35; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___lambda__1___closed__39; +static lean_object* l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__1; static lean_object* l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed__42; LEAN_EXPORT lean_object* l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabNoErrorIfUnused__1___closed__2; -static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__12; static lean_object* l_Lean_Elab_Term_Quotation___aux__Lean__Elab__Quotation______macroRules__Lean__Elab__Term__Quotation__commandElab__stx__quot____1___closed__30; 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*); static lean_object* l_Lean_Elab_Term_Quotation_instReprMatchResult___closed__10; LEAN_EXPORT lean_object* l_Lean_resolveNamespaceCore___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__26___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_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___lambda__2___closed__21; +LEAN_EXPORT lean_object* l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6436_(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_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___lambda__1___closed__6; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__3___closed__21; static lean_object* l_Lean_Elab_Term_Quotation_ArrayStxBuilder_mkNode___closed__61; @@ -772,8 +779,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quota static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__12___closed__1; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getSepStxFromSplice___closed__9; static lean_object* l_Lean_Elab_Term_Quotation_commandElab__stx__quot_____closed__11; -LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6440____closed__2; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_resolveNamespaceCore___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__26___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_deduplicate(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); @@ -830,8 +836,8 @@ lean_object* l_Lean_Elab_Term_addTermInfo_x27(lean_object*, lean_object*, lean_o static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_floatOutAntiquotTerms___lambda__1___closed__3; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__9___closed__12; LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__20___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6426____closed__2; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__3___closed__17; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__2___closed__9; static lean_object* l___private_Init_Meta_0__Lean_quoteList___at_Lean_Elab_Term_Quotation_ArrayStxBuilder_build___spec__2___closed__6; uint8_t l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_365____spec__1(lean_object*, lean_object*); @@ -845,9 +851,9 @@ uint8_t l_Lean_Syntax_isQuot(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__2___closed__11; LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_deduplicate___lambda__3(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__14___closed__20; +static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__11; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__24___closed__2; static lean_object* l_Lean_Elab_Term_Quotation_instQuotePreresolvedMkStr1__lean___closed__10; -static lean_object* l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__2; static lean_object* l_Lean_Elab_Term_Quotation_instReprMatchResult___closed__13; static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__3___closed__3; static lean_object* l_Lean_Elab_Term_Quotation_mkTuple___closed__16; @@ -868,6 +874,7 @@ static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_ static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__23___closed__18; LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_findUsedAlts_go___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__61; +static lean_object* l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__3; lean_object* l___private_Init_Meta_0__Lean_getEscapedNameParts_x3f(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_Quotation_ArrayStxBuilder_mkNode___closed__35; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__14___closed__5; @@ -880,6 +887,7 @@ static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_ uint8_t l_Lean_Name_isAtomic(lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__17(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_throwErrorAt___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__24(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__10; lean_object* lean_string_length(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_floatOutAntiquotTerms___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_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__7(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -889,7 +897,6 @@ static lean_object* l_Lean_Elab_Term_Quotation_instQuotePreresolvedMkStr1__lean_ static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getSepStxFromSplice___closed__11; static lean_object* l_List_foldlM___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__17___closed__6; lean_object* l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6419_(lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_Quotation_ArrayStxBuilder_mkNode___closed__5; LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_compileStxMatch___spec__5___lambda__1(lean_object*, lean_object*, lean_object*); @@ -897,10 +904,8 @@ static lean_object* l_Lean_Elab_Term_Quotation_ArrayStxBuilder_mkNode___closed__ static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__22; static lean_object* l_Lean_Elab_Term_Quotation_ArrayStxBuilder_mkNode___closed__64; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__27___closed__7; -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412_(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___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_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__62; -static lean_object* l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__8; lean_object* l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__28___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_SepArray_ofElems(lean_object*, lean_object*); @@ -918,10 +923,12 @@ static lean_object* l_Lean_Elab_Term_Quotation_getQuotKind___closed__7; static lean_object* l_Lean_Elab_Term_Quotation_ArrayStxBuilder_mkNode___closed__39; static lean_object* l_List_forIn_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_compileStxMatch___spec__4___closed__8; LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_compileStxMatch___spec__3(lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__3; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___lambda__1___closed__21; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__15; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___lambda__2___closed__22; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___lambda__2___closed__8; +static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6429____closed__2; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___closed__2; static lean_object* l_Lean_Elab_Term_Quotation_instQuotePreresolvedMkStr1__lean___closed__19; static lean_object* l_Lean_Elab_Term_Quotation___aux__Lean__Elab__Quotation______macroRules__Lean__Elab__Term__Quotation__commandElab__stx__quot____1___closed__54; @@ -930,7 +937,6 @@ static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_ lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed__8; static lean_object* l___private_Init_Meta_0__Lean_quoteList___at_Lean_Elab_Term_Quotation_ArrayStxBuilder_build___spec__2___closed__5; -static lean_object* l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__4; static lean_object* l_Lean_Elab_Term_Quotation_instQuotePreresolvedMkStr1__lean___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__10(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -964,7 +970,6 @@ static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_ static lean_object* l_Lean_Elab_Term_Quotation_instReprMatchResult___closed__12; lean_object* l_StateRefT_x27_lift(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_Quotation_instReprMatchResult___closed__9; -static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__11; LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__13(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__35; static lean_object* l_Lean_Elab_Term_Quotation_ArrayStxBuilder_mkNode___closed__7; @@ -974,7 +979,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quota lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__13___rarg(lean_object*); static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__11___closed__3; static lean_object* l_Lean_Elab_Term_Quotation_mkTuple___closed__12; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed__18; lean_object* l_Substring_prevn(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_Quotation_mkTuple___closed__10; @@ -983,7 +987,6 @@ lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMe LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_mapM_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__4___closed__2; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_deduplicate___lambda__1___closed__2; -static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__7; uint64_t lean_uint64_xor(uint64_t, uint64_t); LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_quoteList___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__29(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_markRhss___spec__6___lambda__1___closed__1; @@ -998,7 +1001,6 @@ LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_Quotation_match__ static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_floatOutAntiquotTerms___lambda__1___closed__11; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__11___closed__6; -static lean_object* l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__3; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__14(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_markRhss___spec__6___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getSepStxFromSplice___closed__3; @@ -1009,19 +1011,18 @@ static lean_object* l_Lean_Elab_Term_Quotation_ArrayStxBuilder_mkNode___closed__ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___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*); static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getSepStxFromSplice___closed__2; lean_object* l_Lean_Syntax_setInfo(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6440_(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__10___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_compileStxMatch___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___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__3___closed__25; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6422_(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__21___boxed(lean_object**); static lean_object* l_Lean_Elab_Term_Quotation___aux__Lean__Elab__Quotation______macroRules__Lean__Elab__Term__Quotation__commandElab__stx__quot____1___closed__37; static lean_object* l_Lean_Elab_Term_Quotation_getQuotKind___closed__16; lean_object* l_Lean_Syntax_antiquotSpliceKind_x3f(lean_object*); lean_object* l_Array_mkArray1___rarg(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6419____closed__3; static lean_object* l_Lean_Elab_Term_Quotation_mkTuple___closed__13; +static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6436____closed__3; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_Quotation_ArrayStxBuilder_mkNode___closed__53; lean_object* lean_nat_mul(lean_object*, lean_object*); @@ -1033,6 +1034,7 @@ lean_object* l_Lean_Parser_getSyntaxKindOfParserAlias_x3f(lean_object*, lean_obj static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__14___closed__7; LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__23___closed__9; +static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6429____closed__3; static lean_object* l_Lean_Elab_Term_Quotation___aux__Lean__Elab__Quotation______macroRules__Lean__Elab__Term__Quotation__commandElab__stx__quot____1___closed__26; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__25___closed__9; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__25___closed__10; @@ -1059,6 +1061,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_Quotation_resolveSectionVariable(lean_ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___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*); lean_object* l_Array_back___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6443____closed__1; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__10___closed__7; static lean_object* l_Lean_Elab_Term_Quotation_instQuotePreresolvedMkStr1__lean___closed__6; lean_object* l_List_reverse___rarg(lean_object*); @@ -1080,11 +1083,11 @@ static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_ size_t lean_usize_sub(size_t, size_t); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___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_array_mk(lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6419____closed__2; static lean_object* l_Lean_Elab_Term_Quotation_match__syntax_expand___closed__1; uint8_t l_Lean_Syntax_structEq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_resolveNamespaceCore___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__26(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_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6419_(lean_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_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6415_(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6443____closed__3; LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_quoteArray___at_Lean_Elab_Term_Quotation_ArrayStxBuilder_build___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Function_comp___rarg(lean_object*, lean_object*, lean_object*); @@ -1101,16 +1104,14 @@ static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_ static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___lambda__1___closed__36; uint8_t l_Lean_isLitKind(lean_object*); static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__16___closed__3; -static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6426____closed__1; lean_object* l_Lean_logAt___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__8(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_node8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__9; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__23___closed__13; -static lean_object* l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__6; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__2(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_markRhss___spec__6___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__9___closed__5; extern lean_object* l_Lean_instInhabitedName; -static lean_object* l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__7; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getSepStxFromSplice___closed__15; static lean_object* l_Lean_Elab_Term_Quotation_commandElab__stx__quot_____closed__5; LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_compileStxMatch___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*); @@ -1121,7 +1122,6 @@ static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___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_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_compileStxMatch___spec__10(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Init_Meta_0__Lean_quoteArray_go___at_Lean_Elab_Term_Quotation_ArrayStxBuilder_build___spec__3___closed__2; -static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__16; LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_Quotation_match__syntax_expand___spec__10(lean_object*, size_t, size_t); static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__23___closed__4; static lean_object* l_Lean_Elab_Term_Quotation_mkTuple___closed__11; @@ -1157,6 +1157,7 @@ lean_object* l_instDecidableEqNat___boxed(lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__2___closed__8; LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__28(lean_object*, lean_object*); lean_object* lean_string_append(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415_(lean_object*); static lean_object* l_Lean_Elab_Term_Quotation_commandElab__stx__quot_____closed__1; static lean_object* l_Lean_Elab_Term_Quotation_instReprMatchResult___closed__6; LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_compileStxMatch___spec__12(lean_object*, lean_object*, lean_object*, lean_object*); @@ -1198,7 +1199,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quota static lean_object* l___private_Init_Meta_0__Lean_quoteList___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__29___closed__4; extern lean_object* l_Lean_Elab_unsupportedSyntaxExceptionId; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_markRhss___closed__3; -static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__4; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed__28; uint8_t lean_usize_dec_lt(size_t, size_t); @@ -1224,6 +1224,7 @@ lean_object* l_Lean_MessageData_bracket(lean_object*, lean_object*, lean_object* static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__3___closed__30; static lean_object* l___private_Init_Meta_0__Lean_quoteList___at_Lean_Elab_Term_Quotation_ArrayStxBuilder_build___spec__2___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__3___boxed(lean_object**); +static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__5; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__14___closed__13; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__12(lean_object*, size_t, size_t, lean_object*); static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___lambda__1___closed__7; @@ -1231,13 +1232,13 @@ static lean_object* l_Lean_Elab_Term_Quotation_ArrayStxBuilder_mkNode___closed__ static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__10___closed__2; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getSepStxFromSplice___closed__1; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__3___closed__26; -static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6433____closed__2; static lean_object* l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed__23; LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__24___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkConstWithFreshMVarLevels(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_Quotation_match__syntax_expand___spec__3___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_Quotation_getQuotKind___closed__14; LEAN_EXPORT lean_object* l_Lean_Elab_Term_Quotation_instReprMatchResult___boxed(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__6; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__14___closed__22; static lean_object* l_Lean_Elab_Term_Quotation___aux__Lean__Elab__Quotation______macroRules__Lean__Elab__Term__Quotation__commandElab__stx__quot____1___closed__53; static lean_object* l_Lean_Elab_Term_Quotation_ArrayStxBuilder_mkNode___closed__41; @@ -1271,6 +1272,7 @@ LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Quotation_0__ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabMatchSyntax_declRange__1(lean_object*); static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_floatOutAntiquotTerms___lambda__1___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_hasNoErrorIfUnused___boxed(lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6422____closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_isAntiquotSplice(lean_object*); size_t lean_usize_land(size_t, size_t); @@ -11403,16 +11405,38 @@ return x_3; static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__42() { _start: { +lean_object* x_1; lean_object* x_2; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__40; +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_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__43() { +_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_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__41; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__42; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__43() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__44() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__41; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__43; +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_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__45() { _start: { lean_object* x_1; @@ -11420,16 +11444,16 @@ x_1 = lean_mk_string_unchecked("TSyntax.raw", 11, 11); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__44() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__46() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__43; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__45; x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__45() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__47() { _start: { lean_object* x_1; @@ -11437,52 +11461,52 @@ x_1 = lean_mk_string_unchecked("TSyntax", 7, 7); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__46() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__48() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__45; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__47; x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__33; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__47() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__49() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_floatOutAntiquotTerms___lambda__1___closed__1; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__45; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__47; x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__33; x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); return x_4; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__48() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__50() { _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_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__47; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__49; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__49() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__51() { _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_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__48; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___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_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__50() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__52() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -11494,19 +11518,19 @@ lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__51() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__53() { _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_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__50; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___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; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__52() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__54() { _start: { lean_object* x_1; @@ -11514,26 +11538,26 @@ x_1 = lean_mk_string_unchecked("x", 1, 1); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__53() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__55() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__52; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__54; x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__54() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__56() { _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_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__52; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__54; 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_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__55() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__57() { _start: { lean_object* x_1; @@ -11541,16 +11565,16 @@ x_1 = lean_mk_string_unchecked("Array.empty.push", 16, 16); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__56() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__58() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__55; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__57; x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__57() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__59() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; @@ -11561,7 +11585,7 @@ x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); return x_4; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__58() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__60() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -11573,31 +11597,31 @@ lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__59() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__61() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__3___closed__32; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__58; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__60; 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_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__60() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__62() { _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_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__59; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__61; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__61() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__63() { _start: { lean_object* x_1; lean_object* x_2; @@ -11606,7 +11630,7 @@ x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__62() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__64() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -11616,7 +11640,7 @@ 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_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__63() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__65() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -11626,31 +11650,31 @@ x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__64() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__66() { _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_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__63; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__65; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__65() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__67() { _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_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__64; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___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; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__66() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__68() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -11662,12 +11686,12 @@ lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__67() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__69() { _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_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__66; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__68; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); @@ -12034,7 +12058,7 @@ lean_inc(x_232); lean_inc(x_237); x_243 = l_Lean_addMacroScope(x_237, x_242, x_232); x_244 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__39; -x_245 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__42; +x_245 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__44; lean_inc(x_231); x_246 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_246, 0, x_231); @@ -12051,12 +12075,12 @@ lean_inc(x_231); x_250 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_250, 0, x_231); lean_ctor_set(x_250, 1, x_249); -x_251 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__46; +x_251 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__48; lean_inc(x_232); lean_inc(x_237); x_252 = l_Lean_addMacroScope(x_237, x_251, x_232); -x_253 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__44; -x_254 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__49; +x_253 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__46; +x_254 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__51; lean_inc(x_231); x_255 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_255, 0, x_231); @@ -12105,18 +12129,18 @@ lean_inc(x_232); lean_inc(x_237); x_276 = l_Lean_addMacroScope(x_237, x_275, x_232); x_277 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__11___closed__2; -x_278 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__51; +x_278 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__53; lean_inc(x_231); x_279 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_279, 0, x_231); lean_ctor_set(x_279, 1, x_277); lean_ctor_set(x_279, 2, x_276); lean_ctor_set(x_279, 3, x_278); -x_280 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__54; +x_280 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__56; lean_inc(x_232); lean_inc(x_237); x_281 = l_Lean_addMacroScope(x_237, x_280, x_232); -x_282 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__53; +x_282 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__55; lean_inc(x_231); x_283 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_283, 0, x_231); @@ -12137,12 +12161,12 @@ lean_inc(x_231); x_289 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_289, 0, x_231); lean_ctor_set(x_289, 1, x_288); -x_290 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__57; +x_290 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__59; lean_inc(x_232); lean_inc(x_237); x_291 = l_Lean_addMacroScope(x_237, x_290, x_232); -x_292 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__56; -x_293 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__60; +x_292 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__58; +x_293 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__62; lean_inc(x_231); x_294 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_294, 0, x_231); @@ -12156,12 +12180,12 @@ lean_inc(x_289); lean_inc(x_274); lean_inc(x_231); x_297 = l_Lean_Syntax_node4(x_231, x_296, x_274, x_287, x_289, x_295); -x_298 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__62; +x_298 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__64; lean_inc(x_232); lean_inc(x_237); x_299 = l_Lean_addMacroScope(x_237, x_298, x_232); -x_300 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__61; -x_301 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__65; +x_300 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__63; +x_301 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__67; lean_inc(x_231); x_302 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_302, 0, x_231); @@ -12175,7 +12199,7 @@ x_304 = l_Lean_Syntax_node1(x_231, x_38, x_303); x_305 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__3___closed__32; x_306 = l_Lean_addMacroScope(x_237, x_305, x_232); x_307 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__3___closed__30; -x_308 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__67; +x_308 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__69; lean_inc(x_231); x_309 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_309, 0, x_231); @@ -12224,7 +12248,7 @@ lean_inc(x_232); lean_inc(x_319); x_325 = l_Lean_addMacroScope(x_319, x_324, x_232); x_326 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__39; -x_327 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__42; +x_327 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__44; lean_inc(x_231); x_328 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_328, 0, x_231); @@ -12241,12 +12265,12 @@ lean_inc(x_231); x_332 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_332, 0, x_231); lean_ctor_set(x_332, 1, x_331); -x_333 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__46; +x_333 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__48; lean_inc(x_232); lean_inc(x_319); x_334 = l_Lean_addMacroScope(x_319, x_333, x_232); -x_335 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__44; -x_336 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__49; +x_335 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__46; +x_336 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__51; lean_inc(x_231); x_337 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_337, 0, x_231); @@ -12295,18 +12319,18 @@ lean_inc(x_232); lean_inc(x_319); x_358 = l_Lean_addMacroScope(x_319, x_357, x_232); x_359 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__11___closed__2; -x_360 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__51; +x_360 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__53; lean_inc(x_231); x_361 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_361, 0, x_231); lean_ctor_set(x_361, 1, x_359); lean_ctor_set(x_361, 2, x_358); lean_ctor_set(x_361, 3, x_360); -x_362 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__54; +x_362 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__56; lean_inc(x_232); lean_inc(x_319); x_363 = l_Lean_addMacroScope(x_319, x_362, x_232); -x_364 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__53; +x_364 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__55; lean_inc(x_231); x_365 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_365, 0, x_231); @@ -12327,12 +12351,12 @@ lean_inc(x_231); x_371 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_371, 0, x_231); lean_ctor_set(x_371, 1, x_370); -x_372 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__57; +x_372 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__59; lean_inc(x_232); lean_inc(x_319); x_373 = l_Lean_addMacroScope(x_319, x_372, x_232); -x_374 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__56; -x_375 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__60; +x_374 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__58; +x_375 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__62; lean_inc(x_231); x_376 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_376, 0, x_231); @@ -12346,12 +12370,12 @@ lean_inc(x_371); lean_inc(x_356); lean_inc(x_231); x_379 = l_Lean_Syntax_node4(x_231, x_378, x_356, x_369, x_371, x_377); -x_380 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__62; +x_380 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__64; lean_inc(x_232); lean_inc(x_319); x_381 = l_Lean_addMacroScope(x_319, x_380, x_232); -x_382 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__61; -x_383 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__65; +x_382 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__63; +x_383 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__67; lean_inc(x_231); x_384 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_384, 0, x_231); @@ -12365,7 +12389,7 @@ x_386 = l_Lean_Syntax_node1(x_231, x_38, x_385); x_387 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__3___closed__32; x_388 = l_Lean_addMacroScope(x_319, x_387, x_232); x_389 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__3___closed__30; -x_390 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__67; +x_390 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__69; lean_inc(x_231); x_391 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_391, 0, x_231); @@ -14394,10 +14418,10 @@ lean_inc(x_217); x_226 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_226, 0, x_217); lean_ctor_set(x_226, 1, x_225); -x_227 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__46; +x_227 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__48; x_228 = l_Lean_addMacroScope(x_223, x_227, x_218); -x_229 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__44; -x_230 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__49; +x_229 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__46; +x_230 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__51; lean_inc(x_217); x_231 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_231, 0, x_217); @@ -14437,10 +14461,10 @@ lean_inc(x_217); x_247 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_247, 0, x_217); lean_ctor_set(x_247, 1, x_246); -x_248 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__46; +x_248 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__48; x_249 = l_Lean_addMacroScope(x_244, x_248, x_218); -x_250 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__44; -x_251 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__49; +x_250 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__46; +x_251 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__51; lean_inc(x_217); x_252 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_252, 0, x_217); @@ -18233,7 +18257,7 @@ static lean_object* _init_l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed_ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__45; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__47; x_2 = l_Lean_Elab_Term_Quotation_mkTuple___closed__4; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; @@ -18244,7 +18268,7 @@ static lean_object* _init_l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed_ { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_floatOutAntiquotTerms___lambda__1___closed__1; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__45; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__47; x_3 = l_Lean_Elab_Term_Quotation_mkTuple___closed__4; x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); return x_4; @@ -19672,7 +19696,7 @@ return x_83; } } } -static lean_object* _init_l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6412____closed__1() { +static lean_object* _init_l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6415____closed__1() { _start: { lean_object* x_1; @@ -19680,16 +19704,16 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Term_Quotation_stxQuot_expand), 8, return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6412_(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_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_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6415_(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { lean_object* x_10; lean_object* x_11; -x_10 = l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6412____closed__1; +x_10 = l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6415____closed__1; x_11 = l_Lean_Elab_Term_adaptExpander(x_10, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); return x_11; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; @@ -19701,7 +19725,7 @@ x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__2() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -19711,47 +19735,47 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__3() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__2; +x_1 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__2; x_2 = l_Lean_Elab_Term_Quotation_commandElab__stx__quot_____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__4() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__3; +x_1 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__3; x_2 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_floatOutAntiquotTerms___lambda__1___closed__3; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__5() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__4; +x_1 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__4; x_2 = l_Lean_Elab_Term_Quotation_commandElab__stx__quot_____closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__6() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__5; +x_1 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__5; x_2 = l_Lean_Elab_Term_Quotation___aux__Lean__Elab__Quotation______macroRules__Lean__Elab__Term__Quotation__commandElab__stx__quot____1___closed__24; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__7() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__7() { _start: { lean_object* x_1; @@ -19759,47 +19783,47 @@ x_1 = lean_mk_string_unchecked("_@", 2, 2); return x_1; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__8() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__6; -x_2 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__7; +x_1 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__6; +x_2 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__7; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__9() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__8; +x_1 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__8; x_2 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_floatOutAntiquotTerms___lambda__1___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__10() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__9; +x_1 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__9; x_2 = l_Lean_Elab_Term_Quotation_commandElab__stx__quot_____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__11() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__10; +x_1 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__10; x_2 = l_Lean_Elab_Term_Quotation_commandElab__stx__quot_____closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__12() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__12() { _start: { lean_object* x_1; @@ -19807,27 +19831,27 @@ x_1 = lean_mk_string_unchecked("_hyg", 4, 4); return x_1; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__13() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__11; -x_2 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__12; +x_1 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__11; +x_2 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__12; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__14() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__13; -x_2 = lean_unsigned_to_nat(6412u); +x_1 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__13; +x_2 = lean_unsigned_to_nat(6415u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__15() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__15() { _start: { lean_object* x_1; @@ -19835,36 +19859,36 @@ x_1 = l_Lean_Elab_Term_termElabAttribute; return x_1; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__16() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__16() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6412_), 9, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6415_), 9, 0); return x_1; } } -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412_(lean_object* x_1) { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415_(lean_object* x_1) { _start: { lean_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_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__15; -x_3 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__1; -x_4 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__14; -x_5 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__16; +x_2 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__15; +x_3 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__1; +x_4 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__14; +x_5 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__16; 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_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6419_(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_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_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6422_(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { lean_object* x_10; lean_object* x_11; -x_10 = l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6412____closed__1; +x_10 = l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6415____closed__1; x_11 = l_Lean_Elab_Term_adaptExpander(x_10, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); return x_11; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6419____closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6422____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; @@ -19876,46 +19900,46 @@ x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6419____closed__2() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6422____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__13; -x_2 = lean_unsigned_to_nat(6419u); +x_1 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__13; +x_2 = lean_unsigned_to_nat(6422u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6419____closed__3() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6422____closed__3() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6419_), 9, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6422_), 9, 0); return x_1; } } -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6419_(lean_object* x_1) { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6422_(lean_object* x_1) { _start: { lean_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_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__15; -x_3 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6419____closed__1; -x_4 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6419____closed__2; -x_5 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6419____closed__3; +x_2 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__15; +x_3 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6422____closed__1; +x_4 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6422____closed__2; +x_5 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6422____closed__3; 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_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6426_(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_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_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6429_(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { lean_object* x_10; lean_object* x_11; -x_10 = l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6412____closed__1; +x_10 = l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6415____closed__1; x_11 = l_Lean_Elab_Term_adaptExpander(x_10, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); return x_11; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6426____closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6429____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; @@ -19927,46 +19951,46 @@ x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6426____closed__2() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6429____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__13; -x_2 = lean_unsigned_to_nat(6426u); +x_1 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__13; +x_2 = lean_unsigned_to_nat(6429u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6426____closed__3() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6429____closed__3() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6426_), 9, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6429_), 9, 0); return x_1; } } -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6426_(lean_object* x_1) { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6429_(lean_object* x_1) { _start: { lean_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_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__15; -x_3 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6426____closed__1; -x_4 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6426____closed__2; -x_5 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6426____closed__3; +x_2 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__15; +x_3 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6429____closed__1; +x_4 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6429____closed__2; +x_5 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6429____closed__3; 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_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6433_(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_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_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6436_(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { lean_object* x_10; lean_object* x_11; -x_10 = l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6412____closed__1; +x_10 = l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6415____closed__1; x_11 = l_Lean_Elab_Term_adaptExpander(x_10, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); return x_11; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6433____closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6436____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; @@ -19978,46 +20002,46 @@ x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6433____closed__2() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6436____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__13; -x_2 = lean_unsigned_to_nat(6433u); +x_1 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__13; +x_2 = lean_unsigned_to_nat(6436u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6433____closed__3() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6436____closed__3() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6433_), 9, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6436_), 9, 0); return x_1; } } -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6433_(lean_object* x_1) { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6436_(lean_object* x_1) { _start: { lean_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_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__15; -x_3 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6433____closed__1; -x_4 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6433____closed__2; -x_5 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6433____closed__3; +x_2 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__15; +x_3 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6436____closed__1; +x_4 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6436____closed__2; +x_5 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6436____closed__3; 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_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6440_(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_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_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6443_(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { lean_object* x_10; lean_object* x_11; -x_10 = l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6412____closed__1; +x_10 = l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6415____closed__1; x_11 = l_Lean_Elab_Term_adaptExpander(x_10, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); return x_11; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6440____closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6443____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; @@ -20029,32 +20053,32 @@ x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6440____closed__2() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6443____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__13; -x_2 = lean_unsigned_to_nat(6440u); +x_1 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__13; +x_2 = lean_unsigned_to_nat(6443u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6440____closed__3() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6443____closed__3() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6440_), 9, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6443_), 9, 0); return x_1; } } -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6440_(lean_object* x_1) { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6443_(lean_object* x_1) { _start: { lean_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_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__15; -x_3 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6440____closed__1; -x_4 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6440____closed__2; -x_5 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6440____closed__3; +x_2 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__15; +x_3 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6443____closed__1; +x_4 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6443____closed__2; +x_5 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6443____closed__3; x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); return x_6; } @@ -20699,7 +20723,7 @@ x_6 = lean_array_uget(x_4, x_3); x_7 = lean_unsigned_to_nat(0u); x_8 = lean_array_uset(x_4, x_3, x_7); x_9 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getSepStxFromSplice___closed__2; -x_10 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__1; +x_10 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__1; x_11 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__3___closed__2; x_12 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__3___closed__3; x_13 = l_Lean_Syntax_node3(x_9, x_10, x_11, x_6, x_12); @@ -21006,7 +21030,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; uint8_t x_10; @@ -21026,7 +21050,7 @@ if (x_14 == 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 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getSepStxFromSplice___closed__2; -x_17 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__1; +x_17 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__1; x_18 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__3___closed__2; x_19 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__3___closed__3; x_20 = l_Lean_Syntax_node3(x_16, x_17, x_18, x_13, x_19); @@ -21052,7 +21076,7 @@ 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 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getSepStxFromSplice___closed__2; -x_30 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__1; +x_30 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__1; x_31 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__3___closed__2; x_32 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__3___closed__3; x_33 = l_Lean_Syntax_node3(x_29, x_30, x_31, x_28, x_32); @@ -26338,53 +26362,53 @@ return x_36; } } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__13(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__13(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -if (lean_obj_tag(x_6) == 2) +if (lean_obj_tag(x_5) == 2) { -lean_object* x_7; lean_object* x_8; uint8_t x_9; -x_7 = lean_ctor_get(x_6, 0); -x_8 = lean_ctor_get(x_6, 1); -x_9 = lean_nat_dec_eq(x_7, x_1); -if (x_9 == 0) +lean_object* x_6; lean_object* x_7; uint8_t x_8; +x_6 = lean_ctor_get(x_5, 0); +x_7 = lean_ctor_get(x_5, 1); +x_8 = lean_nat_dec_eq(x_6, x_1); +if (x_8 == 0) { -lean_object* x_10; -x_10 = lean_box(1); -return x_10; +lean_object* x_9; +x_9 = lean_box(1); +return x_9; } else { -uint8_t x_11; -x_11 = lean_nat_dec_eq(x_8, x_2); -if (x_11 == 0) +uint8_t x_10; +x_10 = lean_nat_dec_eq(x_7, x_2); +if (x_10 == 0) { -lean_object* x_12; -x_12 = lean_box(1); -return x_12; +lean_object* x_11; +x_11 = lean_box(1); +return x_11; } else { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; -x_13 = lean_array_get_size(x_3); -x_14 = lean_mk_empty_array_with_capacity(x_13); -x_15 = lean_unsigned_to_nat(0u); -x_16 = l_Array_mapIdxM_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__6(x_4, x_5, x_1, x_3, x_13, x_15, lean_box(0), x_14); -x_17 = lean_alloc_closure((void*)(l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__11___boxed), 9, 1); -lean_closure_set(x_17, 0, x_16); -x_18 = 1; -x_19 = lean_alloc_ctor(0, 1, 1); -lean_ctor_set(x_19, 0, x_17); -lean_ctor_set_uint8(x_19, sizeof(void*)*1, x_18); -return x_19; +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; +x_12 = lean_array_get_size(x_3); +x_13 = lean_mk_empty_array_with_capacity(x_12); +x_14 = lean_unsigned_to_nat(0u); +x_15 = l_Array_mapFinIdxM_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__6(x_4, x_3, x_1, x_3, x_12, x_14, lean_box(0), x_13); +x_16 = lean_alloc_closure((void*)(l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__11___boxed), 9, 1); +lean_closure_set(x_16, 0, x_15); +x_17 = 1; +x_18 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_18, 0, x_16); +lean_ctor_set_uint8(x_18, sizeof(void*)*1, x_17); +return x_18; } } } else { -lean_object* x_20; -x_20 = lean_box(2); -return x_20; +lean_object* x_19; +x_19 = lean_box(2); +return x_19; } } } @@ -28073,7 +28097,7 @@ lean_inc(x_22); x_51 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_51, 0, x_22); lean_ctor_set(x_51, 1, x_50); -x_52 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__1; +x_52 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__1; lean_inc(x_51); lean_inc(x_22); x_53 = l_Lean_Syntax_node3(x_22, x_52, x_49, x_25, x_51); @@ -28143,9 +28167,9 @@ x_77 = l_Lean_Syntax_node1(x_22, x_2, x_76); lean_inc(x_2); lean_inc(x_22); x_78 = l_Lean_Syntax_node1(x_22, x_2, x_77); -x_79 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__62; +x_79 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__64; x_80 = l_Lean_addMacroScope(x_29, x_79, x_23); -x_81 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__63; +x_81 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__65; lean_inc(x_3); x_82 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_82, 0, x_81); @@ -28153,7 +28177,7 @@ lean_ctor_set(x_82, 1, x_3); x_83 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_83, 0, x_82); lean_ctor_set(x_83, 1, x_3); -x_84 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__61; +x_84 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__63; lean_inc(x_22); x_85 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_85, 0, x_22); @@ -28299,7 +28323,7 @@ lean_inc(x_22); x_139 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_139, 0, x_22); lean_ctor_set(x_139, 1, x_138); -x_140 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__1; +x_140 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__1; lean_inc(x_139); lean_inc(x_22); x_141 = l_Lean_Syntax_node3(x_22, x_140, x_137, x_25, x_139); @@ -28369,9 +28393,9 @@ x_165 = l_Lean_Syntax_node1(x_22, x_2, x_164); lean_inc(x_2); lean_inc(x_22); x_166 = l_Lean_Syntax_node1(x_22, x_2, x_165); -x_167 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__62; +x_167 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__64; x_168 = l_Lean_addMacroScope(x_117, x_167, x_23); -x_169 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__63; +x_169 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__65; lean_inc(x_3); x_170 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_170, 0, x_169); @@ -28379,7 +28403,7 @@ lean_ctor_set(x_170, 1, x_3); x_171 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_171, 0, x_170); lean_ctor_set(x_171, 1, x_3); -x_172 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__61; +x_172 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__63; lean_inc(x_22); x_173 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_173, 0, x_22); @@ -30091,10 +30115,10 @@ x_329 = lean_ctor_get(x_327, 0); lean_inc(x_329); lean_dec(x_327); x_330 = lean_environment_main_module(x_329); -x_331 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__62; +x_331 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__64; lean_inc(x_324); x_332 = l_Lean_addMacroScope(x_330, x_331, x_324); -x_333 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__63; +x_333 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__65; lean_inc(x_2); lean_ctor_set_tag(x_325, 1); lean_ctor_set(x_325, 1, x_2); @@ -30103,7 +30127,7 @@ lean_inc(x_2); x_334 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_334, 0, x_325); lean_ctor_set(x_334, 1, x_2); -x_335 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__61; +x_335 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__63; lean_inc(x_323); x_336 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_336, 0, x_323); @@ -30283,7 +30307,7 @@ x_408 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_408, 0, x_407); lean_ctor_set(x_408, 1, x_356); lean_ctor_set(x_408, 2, x_14); -x_409 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__1; +x_409 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__1; lean_inc(x_379); lean_inc(x_323); x_410 = l_Lean_Syntax_node3(x_323, x_409, x_406, x_408, x_379); @@ -30511,7 +30535,7 @@ x_504 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_504, 0, x_503); lean_ctor_set(x_504, 1, x_452); lean_ctor_set(x_504, 2, x_14); -x_505 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__1; +x_505 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__1; lean_inc(x_475); lean_inc(x_323); x_506 = l_Lean_Syntax_node3(x_323, x_505, x_502, x_504, x_475); @@ -30582,10 +30606,10 @@ x_535 = lean_ctor_get(x_533, 0); lean_inc(x_535); lean_dec(x_533); x_536 = lean_environment_main_module(x_535); -x_537 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__62; +x_537 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__64; lean_inc(x_324); x_538 = l_Lean_addMacroScope(x_536, x_537, x_324); -x_539 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__63; +x_539 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__65; lean_inc(x_2); x_540 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_540, 0, x_539); @@ -30594,7 +30618,7 @@ lean_inc(x_2); x_541 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_541, 0, x_540); lean_ctor_set(x_541, 1, x_2); -x_542 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__61; +x_542 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__63; lean_inc(x_323); x_543 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_543, 0, x_323); @@ -30781,7 +30805,7 @@ x_616 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_616, 0, x_615); lean_ctor_set(x_616, 1, x_564); lean_ctor_set(x_616, 2, x_14); -x_617 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__1; +x_617 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__1; lean_inc(x_587); lean_inc(x_323); x_618 = l_Lean_Syntax_node3(x_323, x_617, x_614, x_616, x_587); @@ -32634,7 +32658,7 @@ x_282 = lean_st_ref_get(x_12, x_13); x_283 = !lean_is_exclusive(x_282); if (x_283 == 0) { -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_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; x_284 = lean_ctor_get(x_282, 0); x_285 = lean_ctor_get(x_284, 0); lean_inc(x_285); @@ -32668,345 +32692,353 @@ lean_inc(x_4); x_298 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_298, 0, x_296); lean_ctor_set(x_298, 1, x_4); +x_299 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__42; lean_inc(x_4); -x_299 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_299, 0, x_298); -lean_ctor_set(x_299, 1, x_4); -x_300 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__39; -lean_inc(x_280); -x_301 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_301, 0, x_280); +x_300 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_300, 0, x_299); +lean_ctor_set(x_300, 1, x_4); +x_301 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_301, 0, x_298); lean_ctor_set(x_301, 1, x_300); -lean_ctor_set(x_301, 2, x_297); -lean_ctor_set(x_301, 3, x_299); -x_302 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__3___closed__11; +x_302 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__39; lean_inc(x_280); -x_303 = lean_alloc_ctor(2, 2, 0); +x_303 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_303, 0, x_280); lean_ctor_set(x_303, 1, x_302); -x_304 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__21; +lean_ctor_set(x_303, 2, x_297); +lean_ctor_set(x_303, 3, x_301); +x_304 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__3___closed__11; lean_inc(x_280); x_305 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_305, 0, x_280); lean_ctor_set(x_305, 1, x_304); -x_306 = l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed__38; +x_306 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__21; +lean_inc(x_280); +x_307 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_307, 0, x_280); +lean_ctor_set(x_307, 1, x_306); +x_308 = l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed__38; lean_inc(x_281); lean_inc(x_286); -x_307 = l_Lean_addMacroScope(x_286, x_306, x_281); -x_308 = l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed__39; -lean_inc(x_4); -x_309 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_309, 0, x_308); -lean_ctor_set(x_309, 1, x_4); -x_310 = l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed__41; +x_309 = l_Lean_addMacroScope(x_286, x_308, x_281); +x_310 = l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed__39; lean_inc(x_4); x_311 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_311, 0, x_310); lean_ctor_set(x_311, 1, x_4); -x_312 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_312, 0, x_309); -lean_ctor_set(x_312, 1, x_311); -x_313 = l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed__37; -lean_inc(x_280); -x_314 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_314, 0, x_280); +x_312 = l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed__41; +lean_inc(x_4); +x_313 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_313, 0, x_312); +lean_ctor_set(x_313, 1, x_4); +x_314 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_314, 0, x_311); lean_ctor_set(x_314, 1, x_313); -lean_ctor_set(x_314, 2, x_307); -lean_ctor_set(x_314, 3, x_312); -x_315 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__20; +x_315 = l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed__37; lean_inc(x_280); -x_316 = l_Lean_Syntax_node2(x_280, x_315, x_305, x_314); -x_317 = l___private_Init_Meta_0__Lean_quoteList___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__22(x_5); +x_316 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_316, 0, x_280); +lean_ctor_set(x_316, 1, x_315); +lean_ctor_set(x_316, 2, x_309); +lean_ctor_set(x_316, 3, x_314); +x_317 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__20; lean_inc(x_280); -x_318 = l_Lean_Syntax_node1(x_280, x_291, x_317); -x_319 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getSepStxFromSplice___closed__6; +x_318 = l_Lean_Syntax_node2(x_280, x_317, x_307, x_316); +x_319 = l___private_Init_Meta_0__Lean_quoteList___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__22(x_5); lean_inc(x_280); -x_320 = l_Lean_Syntax_node2(x_280, x_319, x_316, x_318); -x_321 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__3___closed__17; +x_320 = l_Lean_Syntax_node1(x_280, x_291, x_319); +x_321 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getSepStxFromSplice___closed__6; lean_inc(x_280); -x_322 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_322, 0, x_280); -lean_ctor_set(x_322, 1, x_321); -x_323 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__3___closed__10; -lean_inc(x_322); -lean_inc(x_303); +x_322 = l_Lean_Syntax_node2(x_280, x_321, x_318, x_320); +x_323 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__3___closed__17; lean_inc(x_280); -x_324 = l_Lean_Syntax_node3(x_280, x_323, x_303, x_320, x_322); -x_325 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__25___closed__13; +x_324 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_324, 0, x_280); +lean_ctor_set(x_324, 1, x_323); +x_325 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__3___closed__10; +lean_inc(x_324); +lean_inc(x_305); +lean_inc(x_280); +x_326 = l_Lean_Syntax_node3(x_280, x_325, x_305, x_322, x_324); +x_327 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__25___closed__13; lean_inc(x_281); lean_inc(x_286); -x_326 = l_Lean_addMacroScope(x_286, x_325, x_281); -x_327 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__25___closed__14; +x_328 = l_Lean_addMacroScope(x_286, x_327, x_281); +x_329 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__25___closed__14; lean_inc(x_4); -x_328 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_328, 0, x_327); -lean_ctor_set(x_328, 1, x_4); +x_330 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_330, 0, x_329); +lean_ctor_set(x_330, 1, x_4); lean_inc(x_4); -x_329 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_329, 0, x_328); -lean_ctor_set(x_329, 1, x_4); -x_330 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__25___closed__11; +x_331 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_331, 0, x_330); +lean_ctor_set(x_331, 1, x_4); +x_332 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__25___closed__11; lean_inc(x_280); -x_331 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_331, 0, x_280); -lean_ctor_set(x_331, 1, x_330); -lean_ctor_set(x_331, 2, x_326); -lean_ctor_set(x_331, 3, x_329); -x_332 = l_List_mapM_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__4___closed__10; -x_333 = l_Lean_addMacroScope(x_286, x_332, x_281); -x_334 = l_List_mapM_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__4___closed__9; +x_333 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_333, 0, x_280); +lean_ctor_set(x_333, 1, x_332); +lean_ctor_set(x_333, 2, x_328); +lean_ctor_set(x_333, 3, x_331); +x_334 = l_List_mapM_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__4___closed__10; +x_335 = l_Lean_addMacroScope(x_286, x_334, x_281); +x_336 = l_List_mapM_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__4___closed__9; lean_inc(x_280); -x_335 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_335, 0, x_280); -lean_ctor_set(x_335, 1, x_334); -lean_ctor_set(x_335, 2, x_333); -lean_ctor_set(x_335, 3, x_4); +x_337 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_337, 0, x_280); +lean_ctor_set(x_337, 1, x_336); +lean_ctor_set(x_337, 2, x_335); +lean_ctor_set(x_337, 3, x_4); lean_inc(x_280); -x_336 = l_Lean_Syntax_node1(x_280, x_291, x_335); +x_338 = l_Lean_Syntax_node1(x_280, x_291, x_337); lean_inc(x_280); -x_337 = l_Lean_Syntax_node2(x_280, x_319, x_331, x_336); +x_339 = l_Lean_Syntax_node2(x_280, x_321, x_333, x_338); lean_inc(x_280); -x_338 = l_Lean_Syntax_node3(x_280, x_323, x_303, x_337, x_322); +x_340 = l_Lean_Syntax_node3(x_280, x_325, x_305, x_339, x_324); lean_inc(x_280); -x_339 = l_Lean_Syntax_node2(x_280, x_291, x_324, x_338); +x_341 = l_Lean_Syntax_node2(x_280, x_291, x_326, x_340); lean_inc(x_280); -x_340 = l_Lean_Syntax_node2(x_280, x_319, x_301, x_339); -x_341 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__9___closed__6; +x_342 = l_Lean_Syntax_node2(x_280, x_321, x_303, x_341); +x_343 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__9___closed__6; lean_inc(x_293); lean_inc(x_280); -x_342 = l_Lean_Syntax_node5(x_280, x_341, x_290, x_293, x_293, x_295, x_340); -x_343 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__9___closed__4; +x_344 = l_Lean_Syntax_node5(x_280, x_343, x_290, x_293, x_293, x_295, x_342); +x_345 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__9___closed__4; lean_inc(x_280); -x_344 = l_Lean_Syntax_node1(x_280, x_343, x_342); -x_345 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_floatOutAntiquotTerms___lambda__1___closed__14; +x_346 = l_Lean_Syntax_node1(x_280, x_345, x_344); +x_347 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_floatOutAntiquotTerms___lambda__1___closed__14; lean_inc(x_280); -x_346 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_346, 0, x_280); -lean_ctor_set(x_346, 1, x_345); -x_347 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__9___closed__2; -x_348 = l_Lean_Syntax_node4(x_280, x_347, x_288, x_344, x_346, x_6); -lean_ctor_set(x_282, 0, x_348); +x_348 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_348, 0, x_280); +lean_ctor_set(x_348, 1, x_347); +x_349 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__9___closed__2; +x_350 = l_Lean_Syntax_node4(x_280, x_349, x_288, x_346, x_348, x_6); +lean_ctor_set(x_282, 0, x_350); return x_282; } else { -lean_object* x_349; lean_object* x_350; lean_object* x_351; lean_object* x_352; lean_object* x_353; lean_object* x_354; lean_object* x_355; lean_object* x_356; lean_object* x_357; 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; -x_349 = lean_ctor_get(x_282, 0); -x_350 = lean_ctor_get(x_282, 1); -lean_inc(x_350); -lean_inc(x_349); -lean_dec(x_282); -x_351 = lean_ctor_get(x_349, 0); +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; +x_351 = lean_ctor_get(x_282, 0); +x_352 = lean_ctor_get(x_282, 1); +lean_inc(x_352); lean_inc(x_351); -lean_dec(x_349); -x_352 = lean_environment_main_module(x_351); -x_353 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__9___closed__1; -lean_inc(x_280); -x_354 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_354, 0, x_280); -lean_ctor_set(x_354, 1, x_353); -x_355 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__9___closed__8; +lean_dec(x_282); +x_353 = lean_ctor_get(x_351, 0); +lean_inc(x_353); +lean_dec(x_351); +x_354 = lean_environment_main_module(x_353); +x_355 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__9___closed__1; lean_inc(x_280); -x_356 = l_Lean_Syntax_node1(x_280, x_355, x_3); -x_357 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_floatOutAntiquotTerms___lambda__1___closed__11; -x_358 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_floatOutAntiquotTerms___lambda__1___closed__12; +x_356 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_356, 0, x_280); +lean_ctor_set(x_356, 1, x_355); +x_357 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__9___closed__8; lean_inc(x_280); -x_359 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_359, 0, x_280); -lean_ctor_set(x_359, 1, x_357); -lean_ctor_set(x_359, 2, x_358); -x_360 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_floatOutAntiquotTerms___lambda__1___closed__13; +x_358 = l_Lean_Syntax_node1(x_280, x_357, x_3); +x_359 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_floatOutAntiquotTerms___lambda__1___closed__11; +x_360 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_floatOutAntiquotTerms___lambda__1___closed__12; lean_inc(x_280); -x_361 = lean_alloc_ctor(2, 2, 0); +x_361 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_361, 0, x_280); -lean_ctor_set(x_361, 1, x_360); -x_362 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__40; +lean_ctor_set(x_361, 1, x_359); +lean_ctor_set(x_361, 2, x_360); +x_362 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_floatOutAntiquotTerms___lambda__1___closed__13; +lean_inc(x_280); +x_363 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_363, 0, x_280); +lean_ctor_set(x_363, 1, x_362); +x_364 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__40; lean_inc(x_281); -lean_inc(x_352); -x_363 = l_Lean_addMacroScope(x_352, x_362, x_281); +lean_inc(x_354); +x_365 = l_Lean_addMacroScope(x_354, x_364, x_281); lean_inc(x_4); -x_364 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_364, 0, x_362); -lean_ctor_set(x_364, 1, x_4); +x_366 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_366, 0, x_364); +lean_ctor_set(x_366, 1, x_4); +x_367 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__42; lean_inc(x_4); -x_365 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_365, 0, x_364); -lean_ctor_set(x_365, 1, x_4); -x_366 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__39; -lean_inc(x_280); -x_367 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_367, 0, x_280); -lean_ctor_set(x_367, 1, x_366); -lean_ctor_set(x_367, 2, x_363); -lean_ctor_set(x_367, 3, x_365); -x_368 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__3___closed__11; -lean_inc(x_280); -x_369 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_369, 0, x_280); +x_368 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_368, 0, x_367); +lean_ctor_set(x_368, 1, x_4); +x_369 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_369, 0, x_366); lean_ctor_set(x_369, 1, x_368); -x_370 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__21; +x_370 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__39; lean_inc(x_280); -x_371 = lean_alloc_ctor(2, 2, 0); +x_371 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_371, 0, x_280); lean_ctor_set(x_371, 1, x_370); -x_372 = l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed__38; +lean_ctor_set(x_371, 2, x_365); +lean_ctor_set(x_371, 3, x_369); +x_372 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__3___closed__11; +lean_inc(x_280); +x_373 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_373, 0, x_280); +lean_ctor_set(x_373, 1, x_372); +x_374 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__21; +lean_inc(x_280); +x_375 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_375, 0, x_280); +lean_ctor_set(x_375, 1, x_374); +x_376 = l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed__38; lean_inc(x_281); -lean_inc(x_352); -x_373 = l_Lean_addMacroScope(x_352, x_372, x_281); -x_374 = l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed__39; +lean_inc(x_354); +x_377 = l_Lean_addMacroScope(x_354, x_376, x_281); +x_378 = l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed__39; lean_inc(x_4); -x_375 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_375, 0, x_374); -lean_ctor_set(x_375, 1, x_4); -x_376 = l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed__41; +x_379 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_379, 0, x_378); +lean_ctor_set(x_379, 1, x_4); +x_380 = l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed__41; lean_inc(x_4); -x_377 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_377, 0, x_376); -lean_ctor_set(x_377, 1, x_4); -x_378 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_378, 0, x_375); -lean_ctor_set(x_378, 1, x_377); -x_379 = l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed__37; +x_381 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_381, 0, x_380); +lean_ctor_set(x_381, 1, x_4); +x_382 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_382, 0, x_379); +lean_ctor_set(x_382, 1, x_381); +x_383 = l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed__37; lean_inc(x_280); -x_380 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_380, 0, x_280); -lean_ctor_set(x_380, 1, x_379); -lean_ctor_set(x_380, 2, x_373); -lean_ctor_set(x_380, 3, x_378); -x_381 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__20; +x_384 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_384, 0, x_280); +lean_ctor_set(x_384, 1, x_383); +lean_ctor_set(x_384, 2, x_377); +lean_ctor_set(x_384, 3, x_382); +x_385 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__20; lean_inc(x_280); -x_382 = l_Lean_Syntax_node2(x_280, x_381, x_371, x_380); -x_383 = l___private_Init_Meta_0__Lean_quoteList___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__22(x_5); +x_386 = l_Lean_Syntax_node2(x_280, x_385, x_375, x_384); +x_387 = l___private_Init_Meta_0__Lean_quoteList___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__22(x_5); lean_inc(x_280); -x_384 = l_Lean_Syntax_node1(x_280, x_357, x_383); -x_385 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getSepStxFromSplice___closed__6; +x_388 = l_Lean_Syntax_node1(x_280, x_359, x_387); +x_389 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getSepStxFromSplice___closed__6; lean_inc(x_280); -x_386 = l_Lean_Syntax_node2(x_280, x_385, x_382, x_384); -x_387 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__3___closed__17; +x_390 = l_Lean_Syntax_node2(x_280, x_389, x_386, x_388); +x_391 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__3___closed__17; lean_inc(x_280); -x_388 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_388, 0, x_280); -lean_ctor_set(x_388, 1, x_387); -x_389 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__3___closed__10; -lean_inc(x_388); -lean_inc(x_369); +x_392 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_392, 0, x_280); +lean_ctor_set(x_392, 1, x_391); +x_393 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__3___closed__10; +lean_inc(x_392); +lean_inc(x_373); lean_inc(x_280); -x_390 = l_Lean_Syntax_node3(x_280, x_389, x_369, x_386, x_388); -x_391 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__25___closed__13; +x_394 = l_Lean_Syntax_node3(x_280, x_393, x_373, x_390, x_392); +x_395 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__25___closed__13; lean_inc(x_281); -lean_inc(x_352); -x_392 = l_Lean_addMacroScope(x_352, x_391, x_281); -x_393 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__25___closed__14; +lean_inc(x_354); +x_396 = l_Lean_addMacroScope(x_354, x_395, x_281); +x_397 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__25___closed__14; lean_inc(x_4); -x_394 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_394, 0, x_393); -lean_ctor_set(x_394, 1, x_4); +x_398 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_398, 0, x_397); +lean_ctor_set(x_398, 1, x_4); lean_inc(x_4); -x_395 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_395, 0, x_394); -lean_ctor_set(x_395, 1, x_4); -x_396 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__25___closed__11; -lean_inc(x_280); -x_397 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_397, 0, x_280); -lean_ctor_set(x_397, 1, x_396); -lean_ctor_set(x_397, 2, x_392); -lean_ctor_set(x_397, 3, x_395); -x_398 = l_List_mapM_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__4___closed__10; -x_399 = l_Lean_addMacroScope(x_352, x_398, x_281); -x_400 = l_List_mapM_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__4___closed__9; +x_399 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_399, 0, x_398); +lean_ctor_set(x_399, 1, x_4); +x_400 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__25___closed__11; lean_inc(x_280); x_401 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_401, 0, x_280); lean_ctor_set(x_401, 1, x_400); -lean_ctor_set(x_401, 2, x_399); -lean_ctor_set(x_401, 3, x_4); +lean_ctor_set(x_401, 2, x_396); +lean_ctor_set(x_401, 3, x_399); +x_402 = l_List_mapM_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__4___closed__10; +x_403 = l_Lean_addMacroScope(x_354, x_402, x_281); +x_404 = l_List_mapM_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__4___closed__9; lean_inc(x_280); -x_402 = l_Lean_Syntax_node1(x_280, x_357, x_401); +x_405 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_405, 0, x_280); +lean_ctor_set(x_405, 1, x_404); +lean_ctor_set(x_405, 2, x_403); +lean_ctor_set(x_405, 3, x_4); lean_inc(x_280); -x_403 = l_Lean_Syntax_node2(x_280, x_385, x_397, x_402); +x_406 = l_Lean_Syntax_node1(x_280, x_359, x_405); lean_inc(x_280); -x_404 = l_Lean_Syntax_node3(x_280, x_389, x_369, x_403, x_388); +x_407 = l_Lean_Syntax_node2(x_280, x_389, x_401, x_406); lean_inc(x_280); -x_405 = l_Lean_Syntax_node2(x_280, x_357, x_390, x_404); +x_408 = l_Lean_Syntax_node3(x_280, x_393, x_373, x_407, x_392); lean_inc(x_280); -x_406 = l_Lean_Syntax_node2(x_280, x_385, x_367, x_405); -x_407 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__9___closed__6; -lean_inc(x_359); +x_409 = l_Lean_Syntax_node2(x_280, x_359, x_394, x_408); lean_inc(x_280); -x_408 = l_Lean_Syntax_node5(x_280, x_407, x_356, x_359, x_359, x_361, x_406); -x_409 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__9___closed__4; +x_410 = l_Lean_Syntax_node2(x_280, x_389, x_371, x_409); +x_411 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__9___closed__6; +lean_inc(x_361); lean_inc(x_280); -x_410 = l_Lean_Syntax_node1(x_280, x_409, x_408); -x_411 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_floatOutAntiquotTerms___lambda__1___closed__14; +x_412 = l_Lean_Syntax_node5(x_280, x_411, x_358, x_361, x_361, x_363, x_410); +x_413 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__9___closed__4; lean_inc(x_280); -x_412 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_412, 0, x_280); -lean_ctor_set(x_412, 1, x_411); -x_413 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__9___closed__2; -x_414 = l_Lean_Syntax_node4(x_280, x_413, x_354, x_410, x_412, x_6); -x_415 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_415, 0, x_414); -lean_ctor_set(x_415, 1, x_350); -return x_415; +x_414 = l_Lean_Syntax_node1(x_280, x_413, x_412); +x_415 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_floatOutAntiquotTerms___lambda__1___closed__14; +lean_inc(x_280); +x_416 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_416, 0, x_280); +lean_ctor_set(x_416, 1, x_415); +x_417 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__9___closed__2; +x_418 = l_Lean_Syntax_node4(x_280, x_417, x_356, x_414, x_416, x_6); +x_419 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_419, 0, x_418); +lean_ctor_set(x_419, 1, x_352); +return x_419; } } } else { -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_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_dec(x_18); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_416 = l_Lean_MessageData_ofName(x_17); -x_417 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__15; -x_418 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_418, 0, x_417); -lean_ctor_set(x_418, 1, x_416); -x_419 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__17; -x_420 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_420, 0, x_418); -lean_ctor_set(x_420, 1, x_419); -x_421 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__5; +x_420 = l_Lean_MessageData_ofName(x_17); +x_421 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__15; x_422 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_422, 0, x_421); lean_ctor_set(x_422, 1, x_420); -x_423 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__11; +x_423 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__17; x_424 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_424, 0, x_422); lean_ctor_set(x_424, 1, x_423); -x_425 = l_Lean_throwErrorAt___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__20(x_2, x_424, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -return x_425; +x_425 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__5; +x_426 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_426, 0, x_425); +lean_ctor_set(x_426, 1, x_424); +x_427 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__11; +x_428 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_428, 0, x_426); +lean_ctor_set(x_428, 1, x_427); +x_429 = l_Lean_throwErrorAt___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__20(x_2, x_428, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +return x_429; } } else { -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_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_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_426 = l_Lean_MessageData_ofName(x_17); -x_427 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__15; -x_428 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_428, 0, x_427); -lean_ctor_set(x_428, 1, x_426); -x_429 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__17; -x_430 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_430, 0, x_428); -lean_ctor_set(x_430, 1, x_429); -x_431 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__5; +x_430 = l_Lean_MessageData_ofName(x_17); +x_431 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__15; x_432 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_432, 0, x_431); lean_ctor_set(x_432, 1, x_430); -x_433 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__11; +x_433 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__17; x_434 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_434, 0, x_432); lean_ctor_set(x_434, 1, x_433); -x_435 = l_Lean_throwErrorAt___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__20(x_2, x_434, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -return x_435; +x_435 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__5; +x_436 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_436, 0, x_435); +lean_ctor_set(x_436, 1, x_434); +x_437 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__11; +x_438 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_438, 0, x_436); +lean_ctor_set(x_438, 1, x_437); +x_439 = l_Lean_throwErrorAt___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__20(x_2, x_438, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +return x_439; } } } @@ -34655,6 +34687,7 @@ x_49 = lean_ctor_get(x_20, 0); lean_inc(x_49); lean_dec(x_20); x_50 = l_Lean_Syntax_getNumArgs(x_1); +lean_dec(x_1); x_51 = lean_unsigned_to_nat(1u); x_52 = lean_nat_sub(x_50, x_51); lean_dec(x_50); @@ -34667,12 +34700,11 @@ lean_ctor_set(x_54, 1, x_53); lean_inc(x_2); lean_inc(x_53); lean_inc(x_49); -x_55 = lean_alloc_closure((void*)(l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__13___boxed), 6, 5); +x_55 = lean_alloc_closure((void*)(l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__13___boxed), 5, 4); lean_closure_set(x_55, 0, x_49); lean_closure_set(x_55, 1, x_53); lean_closure_set(x_55, 2, x_16); lean_closure_set(x_55, 3, x_2); -lean_closure_set(x_55, 4, x_1); x_56 = lean_alloc_closure((void*)(l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__14___boxed), 14, 5); lean_closure_set(x_56, 0, x_49); lean_closure_set(x_56, 1, x_2); @@ -35608,11 +35640,11 @@ x_4 = lean_box(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; -x_9 = l_Array_mapIdxM_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Array_mapFinIdxM_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); @@ -35904,18 +35936,17 @@ x_8 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___ return x_8; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_7; -x_7 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__13(x_1, x_2, x_3, x_4, x_5, x_6); -lean_dec(x_6); +lean_object* x_6; +x_6 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__13(x_1, x_2, x_3, x_4, x_5); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -return x_7; +return x_6; } } LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__14___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { @@ -46766,7 +46797,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabMatchSyntax _start: { lean_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_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__15; +x_2 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__15; x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__3___closed__20; x_4 = l___regBuiltin_Lean_Elab_Term_Quotation_elabMatchSyntax__1___closed__2; x_5 = l___regBuiltin_Lean_Elab_Term_Quotation_elabMatchSyntax__1___closed__3; @@ -46942,7 +46973,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabNoErrorIfUn _start: { lean_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_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__15; +x_2 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__15; x_3 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__16___closed__7; x_4 = l___regBuiltin_Lean_Elab_Term_Quotation_elabNoErrorIfUnused__1___closed__2; x_5 = l___regBuiltin_Lean_Elab_Term_Quotation_elabNoErrorIfUnused__1___closed__3; @@ -47052,7 +47083,7 @@ x_4 = l_Lean_addBuiltinDeclarationRanges(x_2, x_3, x_1); return x_4; } } -static lean_object* _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__1() { +static lean_object* _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__1() { _start: { lean_object* x_1; @@ -47060,77 +47091,77 @@ x_1 = lean_mk_string_unchecked("initFn", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__2() { +static lean_object* _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__5; -x_2 = l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__1; +x_1 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__5; +x_2 = l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__3() { +static lean_object* _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__2; -x_2 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__7; +x_1 = l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__2; +x_2 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__7; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__4() { +static lean_object* _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__3; +x_1 = l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__3; x_2 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_floatOutAntiquotTerms___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_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__5() { +static lean_object* _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__4; +x_1 = l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__4; x_2 = l_Lean_Elab_Term_Quotation_commandElab__stx__quot_____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__6() { +static lean_object* _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__5; +x_1 = l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__5; x_2 = l_Lean_Elab_Term_Quotation_commandElab__stx__quot_____closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__7() { +static lean_object* _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__6; -x_2 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__12; +x_1 = l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__6; +x_2 = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__12; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__8() { +static lean_object* _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__7; -x_2 = lean_unsigned_to_nat(16962u); +x_1 = l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__7; +x_2 = lean_unsigned_to_nat(16968u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__9() { +static lean_object* _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__9() { _start: { lean_object* x_1; @@ -47138,24 +47169,24 @@ x_1 = lean_mk_string_unchecked("alt", 3, 3); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__10() { +static lean_object* _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Elab_Term_Quotation_commandElab__stx__quot_____closed__1; x_2 = l_List_forIn_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_compileStxMatch___spec__4___closed__1; -x_3 = l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__9; +x_3 = l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__9; x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968_(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; x_2 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_compileStxMatch___closed__1; x_3 = 0; -x_4 = l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__8; +x_4 = l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__8; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); if (lean_obj_tag(x_5) == 0) { @@ -47163,7 +47194,7 @@ lean_object* x_6; lean_object* x_7; uint8_t x_8; lean_object* x_9; x_6 = lean_ctor_get(x_5, 1); lean_inc(x_6); lean_dec(x_5); -x_7 = l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__10; +x_7 = l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__10; x_8 = 1; x_9 = l_Lean_registerTraceClass(x_7, x_8, x_4, x_6); if (lean_obj_tag(x_9) == 0) @@ -47891,6 +47922,10 @@ l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Qu lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__66); l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__67 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__67(); lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__67); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__68 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__68(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__68); +l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__69 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__69(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___closed__69); l_Lean_resolveNamespaceCore___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__26___closed__1 = _init_l_Lean_resolveNamespaceCore___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__26___closed__1(); lean_mark_persistent(l_Lean_resolveNamespaceCore___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__26___closed__1); l_Lean_resolveNamespaceCore___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__26___closed__2 = _init_l_Lean_resolveNamespaceCore___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__26___closed__2(); @@ -48303,77 +48338,77 @@ l_Lean_Elab_Term_Quotation___aux__Lean__Elab__Quotation______macroRules__Lean__E lean_mark_persistent(l_Lean_Elab_Term_Quotation___aux__Lean__Elab__Quotation______macroRules__Lean__Elab__Term__Quotation__commandElab__stx__quot____1___closed__55); l_Lean_Elab_Term_Quotation___aux__Lean__Elab__Quotation______macroRules__Lean__Elab__Term__Quotation__commandElab__stx__quot____1___closed__56 = _init_l_Lean_Elab_Term_Quotation___aux__Lean__Elab__Quotation______macroRules__Lean__Elab__Term__Quotation__commandElab__stx__quot____1___closed__56(); lean_mark_persistent(l_Lean_Elab_Term_Quotation___aux__Lean__Elab__Quotation______macroRules__Lean__Elab__Term__Quotation__commandElab__stx__quot____1___closed__56); -l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6412____closed__1 = _init_l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6412____closed__1(); -lean_mark_persistent(l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6412____closed__1); -l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__1 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__1(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__1); -l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__2 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__2(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__2); -l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__3 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__3(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__3); -l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__4 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__4(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__4); -l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__5 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__5(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__5); -l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__6 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__6(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__6); -l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__7 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__7(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__7); -l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__8 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__8(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__8); -l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__9 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__9(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__9); -l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__10 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__10(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__10); -l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__11 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__11(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__11); -l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__12 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__12(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__12); -l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__13 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__13(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__13); -l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__14 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__14(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__14); -l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__15 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__15(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__15); -l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__16 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__16(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412____closed__16); -if (builtin) {res = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6412_(lean_io_mk_world()); +l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6415____closed__1 = _init_l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6415____closed__1(); +lean_mark_persistent(l_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_6415____closed__1); +l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__1 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__1); +l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__2 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__2); +l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__3 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__3); +l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__4 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__4(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__4); +l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__5 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__5(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__5); +l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__6 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__6(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__6); +l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__7 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__7(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__7); +l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__8 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__8(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__8); +l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__9 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__9(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__9); +l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__10 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__10(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__10); +l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__11 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__11(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__11); +l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__12 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__12(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__12); +l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__13 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__13(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__13); +l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__14 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__14(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__14); +l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__15 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__15(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__15); +l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__16 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__16(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415____closed__16); +if (builtin) {res = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6415_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6419____closed__1 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6419____closed__1(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6419____closed__1); -l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6419____closed__2 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6419____closed__2(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6419____closed__2); -l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6419____closed__3 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6419____closed__3(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6419____closed__3); -if (builtin) {res = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6419_(lean_io_mk_world()); +}l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6422____closed__1 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6422____closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6422____closed__1); +l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6422____closed__2 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6422____closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6422____closed__2); +l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6422____closed__3 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6422____closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6422____closed__3); +if (builtin) {res = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6422_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6426____closed__1 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6426____closed__1(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6426____closed__1); -l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6426____closed__2 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6426____closed__2(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6426____closed__2); -l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6426____closed__3 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6426____closed__3(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6426____closed__3); -if (builtin) {res = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6426_(lean_io_mk_world()); +}l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6429____closed__1 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6429____closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6429____closed__1); +l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6429____closed__2 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6429____closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6429____closed__2); +l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6429____closed__3 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6429____closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6429____closed__3); +if (builtin) {res = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6429_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6433____closed__1 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6433____closed__1(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6433____closed__1); -l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6433____closed__2 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6433____closed__2(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6433____closed__2); -l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6433____closed__3 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6433____closed__3(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6433____closed__3); -if (builtin) {res = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6433_(lean_io_mk_world()); +}l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6436____closed__1 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6436____closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6436____closed__1); +l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6436____closed__2 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6436____closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6436____closed__2); +l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6436____closed__3 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6436____closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6436____closed__3); +if (builtin) {res = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6436_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6440____closed__1 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6440____closed__1(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6440____closed__1); -l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6440____closed__2 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6440____closed__2(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6440____closed__2); -l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6440____closed__3 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6440____closed__3(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6440____closed__3); -if (builtin) {res = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6440_(lean_io_mk_world()); +}l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6443____closed__1 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6443____closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6443____closed__1); +l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6443____closed__2 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6443____closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6443____closed__2); +l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6443____closed__3 = _init_l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6443____closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6443____closed__3); +if (builtin) {res = l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6443_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l_Lean_Elab_Term_Quotation_instReprMatchResult___closed__1 = _init_l_Lean_Elab_Term_Quotation_instReprMatchResult___closed__1(); @@ -48858,27 +48893,27 @@ lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_Quotation_elabNoErrorIfUnused if (builtin) {res = l___regBuiltin_Lean_Elab_Term_Quotation_elabNoErrorIfUnused_declRange__1(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__1 = _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__1(); -lean_mark_persistent(l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__1); -l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__2 = _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__2(); -lean_mark_persistent(l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__2); -l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__3 = _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__3(); -lean_mark_persistent(l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__3); -l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__4 = _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__4(); -lean_mark_persistent(l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__4); -l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__5 = _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__5(); -lean_mark_persistent(l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__5); -l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__6 = _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__6(); -lean_mark_persistent(l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__6); -l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__7 = _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__7(); -lean_mark_persistent(l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__7); -l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__8 = _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__8(); -lean_mark_persistent(l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__8); -l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__9 = _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__9(); -lean_mark_persistent(l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__9); -l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__10 = _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__10(); -lean_mark_persistent(l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__10); -if (builtin) {res = l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962_(lean_io_mk_world()); +}l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__1 = _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__1(); +lean_mark_persistent(l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__1); +l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__2 = _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__2(); +lean_mark_persistent(l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__2); +l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__3 = _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__3(); +lean_mark_persistent(l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__3); +l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__4 = _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__4(); +lean_mark_persistent(l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__4); +l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__5 = _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__5(); +lean_mark_persistent(l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__5); +l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__6 = _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__6(); +lean_mark_persistent(l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__6); +l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__7 = _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__7(); +lean_mark_persistent(l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__7); +l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__8 = _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__8(); +lean_mark_persistent(l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__8); +l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__9 = _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__9(); +lean_mark_persistent(l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__9); +l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__10 = _init_l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__10(); +lean_mark_persistent(l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968____closed__10); +if (builtin) {res = l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16968_(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/StructInst.c b/stage0/stdlib/Lean/Elab/StructInst.c index 09b45eca86c1..9b8985352ce0 100644 --- a/stage0/stdlib/Lean/Elab/StructInst.c +++ b/stage0/stdlib/Lean/Elab/StructInst.c @@ -33,8 +33,8 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_isDefaultMiss LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_expandNonAtomicExplicitSources___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_EXPORT lean_object* l_Lean_Elab_Term_StructInst_mkProjStx_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_tryToSynthesizeDefault_loop(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688_(lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_getFieldIdx___lambda__1(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__11; static lean_object* l___regBuiltin_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev_declRange__1___closed__1; LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStructInstAux___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_Struct_structName___boxed(lean_object*); @@ -55,6 +55,7 @@ lean_object* l_Lean_mkAppN(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_isDefaultMissing_x3f___rarg___lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_expandCompositeFields___lambda__1(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_toFieldLHS(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__10; LEAN_EXPORT lean_object* l_List_foldlM___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStruct___spec__5___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_expandNonAtomicExplicitSources_go___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_mkDefaultValueAux_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -147,7 +148,6 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Stru LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_mkFieldMap___spec__4___boxed(lean_object*, lean_object*); static lean_object* l_List_mapM_loop___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_expandNumLitFields___spec__3___closed__5; lean_object* l_Lean_findField_x3f(lean_object*, lean_object*, lean_object*); -uint8_t l_Array_contains___at_Lean_findField_x3f___spec__1(lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Elab_Term_StructInst_DefaultFields_allDefaultMissing_go___spec__5___rarg___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_mkFieldMap___spec__4(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStructInstAux___spec__1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -184,16 +184,18 @@ lean_object* lean_array_fget(lean_object*, lean_object*); lean_object* l_Lean_Meta_forallTelescope___at_Lean_Meta_mapForallTelescope_x27___spec__1___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_mkDefaultValueAux_x3f___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__2; static lean_object* l_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev___lambda__1___closed__6; LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_toFieldLHS___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_isDefaultMissing_x3f___at_Lean_Elab_Term_StructInst_DefaultFields_allDefaultMissing_go___spec__1___rarg___lambda__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___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_Elab_StructInst_0__Lean_Elab_Term_StructInst_groupFields___spec__2(size_t, size_t, lean_object*); lean_object* l_Lean_Syntax_TSepArray_getElems___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_isModifyOp_x3f___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Macro_throwError___rarg(lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Expr_fvarId_x21(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_findDefaultMissing_x3f(lean_object*); LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_mkStructView___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_isDefaultMissing_x3f___at_Lean_Elab_Term_StructInst_DefaultFields_propagateLoop___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*); @@ -227,7 +229,7 @@ LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_StructInst static lean_object* l_List_format___at_Lean_Elab_Term_StructInst_formatStruct___spec__3___closed__1; lean_object* l_Lean_stringToMessageData(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_Struct_structName(lean_object*); -static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__8; +lean_object* l_Lean_LocalDecl_setValue(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_getStructSource___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev___lambda__1___closed__2; uint8_t l___private_Lean_Util_Trace_0__Lean_checkTraceOption(lean_object*, lean_object*, lean_object*); @@ -260,13 +262,13 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_isDefaultMiss static lean_object* l___regBuiltin_Lean_Elab_Term_StructInst_expandStructInstExpectedType__1___closed__8; LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___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_List_format___at_Lean_Elab_Term_StructInst_formatStruct___spec__3___closed__4; +lean_object* l_Lean_LocalDecl_index(lean_object*); static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_getStructName___closed__2; LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_mkStructView___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_mkFieldMap___spec__7(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_getStructureFields(lean_object*, lean_object*); extern lean_object* l_instInhabitedPUnit; lean_object* l_Lean_Meta_project_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__14; lean_object* l_Lean_getDefaultFnForField_x3f(lean_object*, lean_object*, lean_object*); static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_isModifyOp_x3f___spec__3___closed__1; static lean_object* l_List_mapM_loop___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_groupFields___spec__6___closed__1; @@ -276,6 +278,7 @@ static lean_object* l___regBuiltin_Lean_Elab_Term_StructInst_elabStructInst_decl LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStruct___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isLambda(lean_object*); static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_expandNonAtomicExplicitSources_go___lambda__1___closed__4; +lean_object* l_Lean_PersistentArray_set___rarg(lean_object*, lean_object*, lean_object*); size_t lean_ptr_addr(lean_object*); lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); static lean_object* l_List_foldlM___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStruct___spec__5___closed__2; @@ -300,20 +303,18 @@ static lean_object* l_Lean_Elab_Term_StructInst_instInhabitedField___closed__1; lean_object* l_Lean_Meta_mkFreshLevelMVars(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_getFieldValue_x3f(lean_object*, lean_object*); static lean_object* l_List_foldlM___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStruct___spec__5___lambda__1___closed__4; -static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__13; LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStructInstAux___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_instInhabitedField(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_expandNonAtomicExplicitSources___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__9; static lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_mkDefaultValueAux_x3f___closed__3; static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_getStructSource___spec__2___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__7; LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_Term_StructInst_formatField___spec__3(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_findDefaultMissing_x3f___at_Lean_Elab_Term_StructInst_DefaultFields_propagateLoop___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Elab_Term_StructInst_DefaultFields_propagateLoop___spec__16(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_mkFieldMap___closed__2; static lean_object* l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__11; +lean_object* lean_local_ctx_find(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_markDefaultMissing(lean_object*); static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_expandCompositeFields___closed__1; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStructInstAux___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -324,6 +325,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_getFieldName_ static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_expandNonAtomicExplicitSources_go___lambda__1___closed__2; lean_object* l_liftExcept___at_Lean_Elab_liftMacroM___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_expandNumLitFields___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_StructInst_DefaultFields_mkDefaultValueAux_x3f___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_expandCompositeFields___spec__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_StructInst_instInhabitedSource___closed__1; @@ -331,10 +333,9 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_isRoundDone__ lean_object* l_Lean_Elab_expandMacroImpl_x3f(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_FieldLHS_toSyntax___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Term_StructInst_DefaultFields_allDefaultMissing_go___spec__5___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Array_contains___at_Lean_findField_x3f___spec__1___boxed(lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_synthesizeAppInstMVars(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_groupFields(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__1; +lean_object* l_Lean_PersistentHashMap_insert___at_Lean_LocalContext_mkLocalDecl___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_groupFields___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_ResolveName_resolveNamespace(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev_declRange__1___closed__6; @@ -367,6 +368,7 @@ lean_object* l_Lean_mkHole(lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_instToFormatStruct; static lean_object* l_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev___lambda__1___closed__7; static lean_object* l_List_mapM_loop___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_expandParentFields___spec__3___closed__2; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___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* l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_allDefaultMissing___at_Lean_Elab_Term_StructInst_DefaultFields_propagateLoop___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_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStructInstAux___spec__4___closed__5; @@ -378,6 +380,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_Struct_setParams(lean_objec LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_reduce___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_lambdaLetTelescope___at___private_Lean_Meta_InferType_0__Lean_Meta_inferLambdaType___spec__1___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_mapM_loop___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_groupFields___spec__6___closed__2; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___spec__4(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_elabTerm___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Term_StructInst_DefaultFields_allDefaultMissing_go___spec__5___rarg___lambda__4(lean_object*, lean_object*); @@ -466,11 +469,13 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_instInhabitedExplicitSource LEAN_EXPORT lean_object* l_Array_filterMapM___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_groupFields___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_StructInst_throwFailedToElabField___rarg___closed__2; static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStruct___closed__3; +static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__4; static lean_object* l___regBuiltin_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev_declRange__1___closed__5; static lean_object* l___regBuiltin_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_getHierarchyDepth(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_mkProjStx_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_StructInst_formatStruct___closed__9; +static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__14; static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_getStructName___lambda__1___closed__1; static lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_mkDefaultValueAux_x3f___closed__5; static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_expandNonAtomicExplicitSources_go___lambda__1___closed__10; @@ -500,6 +505,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_propagateLoop LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_addMissingFields___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_mkFieldMap___spec__5___boxed(lean_object*, lean_object*); uint8_t lean_name_eq(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_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_isModifyOp_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_Lean_Elab_liftMacroM___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStructInstAux___spec__1___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); @@ -518,6 +524,7 @@ static lean_object* l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___c LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_instToStringFieldStruct; LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_mkFieldMap___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___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_groupFields___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_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__13; lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_mkDefaultValueAux_x3f___closed__2; static lean_object* l_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev___lambda__1___closed__5; @@ -541,9 +548,11 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_Stru uint8_t l_Lean_Syntax_isIdent(lean_object*); static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__21; static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_expandNonAtomicExplicitSources_go___lambda__1___closed__7; +lean_object* l_Lean_LocalDecl_fvarId(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_expandNonAtomicExplicitSources(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_Field_isSimple(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_mkFieldMap___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___spec__3___closed__2; lean_object* l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_ensureType___spec__1___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_mkFieldMap___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_format___at_Lean_Elab_Term_StructInst_formatStruct___spec__3___closed__5; @@ -551,6 +560,7 @@ lean_object* l_Lean_Elab_Term_mkTacticMVar(lean_object*, lean_object*, lean_obje lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_withSynthesizeImp___rarg(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_foldlM___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStruct___spec__5___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_StructInst_formatStruct___spec__2___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___spec__3___closed__1; extern lean_object* l_Std_Format_defWidth; static lean_object* l___regBuiltin_Lean_Elab_Term_StructInst_elabStructInst_declRange__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_allDefaultMissing___at_Lean_Elab_Term_StructInst_DefaultFields_propagateLoop___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -569,6 +579,7 @@ LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_Term_StructInst_formatField lean_object* l_Lean_MVarId_assign___at_Lean_Elab_Term_exprToSyntax___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__7; static lean_object* l_List_mapM_loop___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_expandNumLitFields___spec__3___closed__6; +lean_object* l_Lean_Meta_instInhabitedMetaM___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStructInstAux___spec__5___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_instToStringStruct; lean_object* l_Lean_MessageData_ofConstName(lean_object*); @@ -588,6 +599,7 @@ static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructIns static lean_object* l___regBuiltin_Lean_Elab_Term_StructInst_expandStructInstExpectedType__1___closed__1; static lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStructInstAux___spec__4___closed__4; lean_object* l_List_tail_x21___rarg(lean_object*); +static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__11; LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_mkCtorHeader(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_StructInst_0__Lean_Elab_Term_StructInst_getFieldIdx___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_throwFailedToElabField___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -610,6 +622,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_isDefaultMiss static lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStructInstAux___spec__5___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_isDefaultMissing_x3f___at_Lean_Elab_Term_StructInst_DefaultFields_allDefaultMissing_go___spec__1(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_StructInst_expandStructInstExpectedType_declRange__1___closed__6; +static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__12; static lean_object* l_Lean_Elab_Term_StructInst_formatField___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_getFieldIdx(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_MVarId_isAssigned___at_Lean_Elab_Term_StructInst_DefaultFields_allDefaultMissing_go___spec__2___rarg___lambda__1(lean_object*, lean_object*, lean_object*); @@ -624,6 +637,7 @@ static lean_object* l___regBuiltin_Lean_Elab_Term_StructInst_elabStructInst__1__ LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_Struct_modifyFieldsM___at_Lean_Elab_Term_StructInst_Struct_modifyFields___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_MVarId_isAssigned___at_Lean_Elab_Term_StructInst_DefaultFields_propagateLoop___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_StructInst_DefaultFields_propagateLoop___spec__4___closed__1; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___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___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_isSimpleField_x3f___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_step(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__7; @@ -641,7 +655,7 @@ static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructIns LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_isDefaultMissing_x3f___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev_declRange__1___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_StructInst_expandStructInstExpectedType__1(lean_object*); -static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__4; +static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__6; static lean_object* l_List_foldlM___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStruct___spec__5___closed__4; static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_getStructSource___spec__2___closed__4; static lean_object* l_List_format___at_Lean_Elab_Term_StructInst_formatStruct___spec__3___closed__2; @@ -662,7 +676,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_isDefaultMiss lean_object* l_Lean_Syntax_SepArray_ofElems(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_getStructName___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_elabStructInst(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__12; uint8_t lean_nat_dec_lt(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_StructInst_instToStringStruct___closed__1; lean_object* lean_environment_main_module(lean_object*); @@ -672,9 +685,9 @@ static lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_tryToSynthesizeDef static lean_object* l___regBuiltin_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev_declRange__1___closed__4; LEAN_EXPORT lean_object* l_List_findSomeM_x3f___at_Lean_Elab_Term_StructInst_DefaultFields_findDefaultMissing_x3f___spec__1___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_Struct_source(lean_object*); +lean_object* l_Lean_Meta_getLocalInstances(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__14; static lean_object* l_List_mapM_loop___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_expandNumLitFields___spec__3___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_mkProjStx_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); static lean_object* l_List_foldlM___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_mkFieldMap___spec__10___closed__4; @@ -708,6 +721,7 @@ static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_StructInst_expand static lean_object* l_Lean_Elab_Term_StructInst_formatStruct___closed__5; static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___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*); +uint8_t l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__6; static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_getStructName_throwUnexpectedExpectedType___closed__4; LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Elab_Term_StructInst_DefaultFields_propagateLoop___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*); @@ -736,6 +750,7 @@ static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructIns static lean_object* l_Lean_Elab_Term_StructInst_FieldVal_toSyntax___closed__2; static lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_propagateLoop___closed__3; lean_object* l_Lean_Expr_getAppFn(lean_object*); +lean_object* l_Lean_Meta_withLCtx___at___private_Lean_Meta_Basic_0__Lean_Meta_mkLevelErrorMessageCore___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_isStructure(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_StructInst_elabStructInst___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev___spec__2(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); @@ -743,13 +758,16 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_StructInst_throwF lean_object* l_Array_mkArray1___rarg(lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_StructInst_expandStructInstExpectedType_declRange__1(lean_object*); lean_object* lean_nat_mul(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_Struct_setFields(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_Term_StructInst_DefaultFields_tryToSynthesizeDefault_loop___lambda__1(lean_object*); +static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__8; LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_getStructName_throwUnknownExpectedType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_mkStructView___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_Term_StructInst_Struct_allDefault___lambda__1(lean_object*); static lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_propagateLoop___closed__4; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev___spec__2___closed__5; +static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__9; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_groupFields___spec__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_mkStructView(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_mkCtorHeaderAux___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -776,7 +794,6 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_StructInst_0 LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_tryToSynthesizeDefault___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_isDefaultMissing_x3f(lean_object*); lean_object* l_String_intercalate(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__6; size_t lean_usize_sub(size_t, size_t); lean_object* lean_array_mk(lean_object*); static lean_object* l_Lean_Elab_Term_StructInst_instInhabitedStruct___closed__1; @@ -803,6 +820,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_StructInst_elabStructInst LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStructInstAux___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Elab_Util_0__Lean_Elab_evalSyntaxConstantUnsafe(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev___lambda__1___closed__8; +static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__7; static lean_object* l_Lean_Elab_Term_StructInst_Field_toSyntax___closed__1; extern lean_object* l_Lean_instInhabitedName; lean_object* l_Lean_Expr_betaRev(lean_object*, lean_object*, uint8_t, uint8_t); @@ -813,7 +831,6 @@ LEAN_EXPORT lean_object* l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_StructIn LEAN_EXPORT lean_object* l_List_foldlM___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStruct___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_allDefaultMissing_go(lean_object*); size_t lean_array_size(lean_object*); -static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__10; LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStruct___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_reduce(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__23; @@ -822,7 +839,6 @@ static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructIns lean_object* l_instInhabitedOfMonad___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_StructInst_formatStruct___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_mkDefaultValueAux_x3f___lambda__3___boxed(lean_object*); -static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__5; extern lean_object* l_Lean_instInhabitedSyntax; lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStruct___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -838,6 +854,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_trySynthStructInstance_x3f( lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_StructInst_FieldLHS_toSyntax___closed__2; lean_object* l_Lean_MVarId_isAssigned___rarg(lean_object*, lean_object*, lean_object*); +static lean_object* l_panic___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___spec__2___closed__1; static lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_mkDefaultValueAux_x3f___closed__1; static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_getStructSource___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -848,6 +865,7 @@ lean_object* l_Lean_mkAtomFrom(lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_expandParentFields___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_Term_StructInst_Struct_params(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStruct___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_LocalDecl_value_x3f(lean_object*); lean_object* lean_array_get_size(lean_object*); lean_object* l_panic___at___private_Init_Prelude_0__Lean_assembleParts___spec__1(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_expandNumLitFields___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -875,11 +893,11 @@ LEAN_EXPORT lean_object* l_Lean_MVarId_isAssigned___at_Lean_Elab_Term_StructInst LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_404_(uint8_t, uint8_t); static lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStructInstAux___spec__5___rarg___closed__2; -static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__3; -lean_object* l_Lean_Meta_mkLambdaFVars(lean_object*, lean_object*, uint8_t, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_getStructName___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_StructInst_formatStruct___closed__6; +lean_object* l_Array_contains___at_Lean_registerInternalExceptionId___spec__1___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_StructInst_FieldVal_toSyntax___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_groupFields___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Format_joinSep___at_Lean_Elab_Term_StructInst_formatStruct___spec__4(lean_object*, lean_object*); @@ -906,6 +924,7 @@ static lean_object* l___regBuiltin_Lean_Elab_Term_StructInst_elabStructInst_decl lean_object* l_String_toSubstring_x27(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_StructInst_DefaultFields_propagateLoop___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_uset(lean_object*, size_t, lean_object*); +static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__1; lean_object* l_Lean_MessageData_ofName(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_isModifyOp_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*); static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__8; @@ -924,6 +943,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_mkDefaultValu LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_Term_StructInst_formatField___spec__2(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev___lambda__1___closed__11; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_StructInst_throwFailedToElabField___spec__1(lean_object*); +lean_object* l_Lean_LocalContext_findFVar_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_getForallBody(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_propagateExpectedType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__18; @@ -951,6 +971,7 @@ lean_object* l_ReaderT_pure___at_Lean_Elab_liftMacroM___spec__2___rarg___boxed(l LEAN_EXPORT uint8_t l_Lean_Elab_Term_StructInst_Field_isSimple___rarg(lean_object*); static lean_object* l_Lean_Elab_Term_StructInst_formatField___closed__5; static lean_object* l_Lean_Elab_Term_StructInst_mkProjStx_x3f___lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_reduce___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Array_isEmpty___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_MVarId_isAssigned___at_Lean_Elab_Term_StructInst_DefaultFields_allDefaultMissing_go___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__10; @@ -18634,7 +18655,7 @@ 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_findField_x3f___spec__1(x_1, x_6); +x_7 = l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(x_1, x_6); lean_dec(x_6); if (x_7 == 0) { @@ -30125,58 +30146,1290 @@ return x_25; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_reduce___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_panic___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___spec__2___closed__1() { _start: { -lean_object* x_9; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Meta_instInhabitedMetaM___boxed), 5, 1); +lean_closure_set(x_1, 0, lean_box(0)); +return x_1; +} +} +LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = l_panic___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___spec__2___closed__1; +x_8 = lean_panic_fn(x_7, x_1); +x_9 = lean_apply_5(x_8, x_2, x_3, x_4, x_5, x_6); +return x_9; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___spec__3___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean.Elab.Term.StructInst.DefaultFields.reduce", 46, 46); +return x_1; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___spec__3___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_getStructSource___spec__2___closed__1; +x_2 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___spec__3___closed__1; +x_3 = lean_unsigned_to_nat(840u); +x_4 = lean_unsigned_to_nat(42u); +x_5 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_getStructSource___spec__2___closed__3; +x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +uint8_t x_12; +x_12 = lean_usize_dec_lt(x_5, x_4); +if (x_12 == 0) +{ +lean_object* x_13; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_2); +lean_dec(x_1); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_6); +lean_ctor_set(x_13, 1, x_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_3, x_5); +lean_inc(x_6); +x_22 = l_Lean_LocalContext_findFVar_x3f(x_6, x_14); +if (lean_obj_tag(x_22) == 0) +{ +lean_object* x_23; lean_object* x_24; +lean_dec(x_14); +x_23 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___spec__3___closed__2; +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); lean_inc(x_7); +x_24 = l_panic___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___spec__2(x_23, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_24) == 0) +{ +lean_object* x_25; lean_object* x_26; +x_25 = lean_ctor_get(x_24, 1); +lean_inc(x_25); +lean_dec(x_24); +x_26 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_26, 0, x_6); +x_15 = x_26; +x_16 = x_25; +goto block_21; +} +else +{ +uint8_t x_27; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_2); +lean_dec(x_1); +x_27 = !lean_is_exclusive(x_24); +if (x_27 == 0) +{ +return x_24; +} +else +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_24, 0); +x_29 = lean_ctor_get(x_24, 1); +lean_inc(x_29); +lean_inc(x_28); +lean_dec(x_24); +x_30 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +return x_30; +} +} +} +else +{ +uint8_t x_31; +x_31 = !lean_is_exclusive(x_22); +if (x_31 == 0) +{ +lean_object* x_32; lean_object* x_33; +x_32 = lean_ctor_get(x_22, 0); +x_33 = l_Lean_LocalDecl_value_x3f(x_32); +lean_dec(x_32); +if (lean_obj_tag(x_33) == 0) +{ +lean_dec(x_14); +lean_ctor_set(x_22, 0, x_6); +x_15 = x_22; +x_16 = x_11; +goto block_21; +} +else +{ +uint8_t x_34; +lean_free_object(x_22); +x_34 = !lean_is_exclusive(x_33); +if (x_34 == 0) +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_33, 0); +lean_inc(x_1); +x_36 = lean_alloc_closure((void*)(l_Lean_Elab_Term_StructInst_DefaultFields_reduce), 7, 2); +lean_closure_set(x_36, 0, x_1); +lean_closure_set(x_36, 1, x_35); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_2); lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -x_9 = l_Lean_Elab_Term_StructInst_DefaultFields_reduce(x_1, x_3, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_9) == 0) +x_37 = l_Lean_Meta_withLCtx___at___private_Lean_Meta_Basic_0__Lean_Meta_mkLevelErrorMessageCore___spec__2___rarg(x_6, x_2, x_36, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_37) == 0) { -lean_object* x_10; lean_object* x_11; uint8_t x_12; uint8_t x_13; uint8_t x_14; lean_object* x_15; +lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_38 = lean_ctor_get(x_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_fvarId_x21(x_14); +lean_dec(x_14); +x_41 = lean_ctor_get(x_6, 0); +lean_inc(x_41); +x_42 = lean_ctor_get(x_6, 1); +lean_inc(x_42); +lean_inc(x_6); +x_43 = lean_local_ctx_find(x_6, x_40); +if (lean_obj_tag(x_43) == 0) +{ +lean_dec(x_42); +lean_dec(x_41); +lean_dec(x_38); +lean_ctor_set(x_33, 0, x_6); +x_15 = x_33; +x_16 = x_39; +goto block_21; +} +else +{ +uint8_t x_44; +x_44 = !lean_is_exclusive(x_6); +if (x_44 == 0) +{ +lean_object* x_45; lean_object* x_46; uint8_t x_47; +x_45 = lean_ctor_get(x_6, 1); +lean_dec(x_45); +x_46 = lean_ctor_get(x_6, 0); +lean_dec(x_46); +x_47 = !lean_is_exclusive(x_43); +if (x_47 == 0) +{ +lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_48 = lean_ctor_get(x_43, 0); +x_49 = l_Lean_LocalDecl_setValue(x_48, x_38); +x_50 = l_Lean_LocalDecl_fvarId(x_49); +lean_inc(x_49); +x_51 = l_Lean_PersistentHashMap_insert___at_Lean_LocalContext_mkLocalDecl___spec__1(x_41, x_50, x_49); +x_52 = l_Lean_LocalDecl_index(x_49); +lean_ctor_set(x_43, 0, x_49); +x_53 = l_Lean_PersistentArray_set___rarg(x_42, x_52, x_43); +lean_dec(x_52); +lean_ctor_set(x_6, 1, x_53); +lean_ctor_set(x_6, 0, x_51); +lean_ctor_set(x_33, 0, x_6); +x_15 = x_33; +x_16 = x_39; +goto block_21; +} +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; +x_54 = lean_ctor_get(x_43, 0); +lean_inc(x_54); +lean_dec(x_43); +x_55 = l_Lean_LocalDecl_setValue(x_54, x_38); +x_56 = l_Lean_LocalDecl_fvarId(x_55); +lean_inc(x_55); +x_57 = l_Lean_PersistentHashMap_insert___at_Lean_LocalContext_mkLocalDecl___spec__1(x_41, x_56, x_55); +x_58 = l_Lean_LocalDecl_index(x_55); +x_59 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_59, 0, x_55); +x_60 = l_Lean_PersistentArray_set___rarg(x_42, x_58, x_59); +lean_dec(x_58); +lean_ctor_set(x_6, 1, x_60); +lean_ctor_set(x_6, 0, x_57); +lean_ctor_set(x_33, 0, x_6); +x_15 = x_33; +x_16 = x_39; +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_dec(x_6); +x_61 = lean_ctor_get(x_43, 0); +lean_inc(x_61); +if (lean_is_exclusive(x_43)) { + lean_ctor_release(x_43, 0); + x_62 = x_43; +} else { + lean_dec_ref(x_43); + x_62 = lean_box(0); +} +x_63 = l_Lean_LocalDecl_setValue(x_61, x_38); +x_64 = l_Lean_LocalDecl_fvarId(x_63); +lean_inc(x_63); +x_65 = l_Lean_PersistentHashMap_insert___at_Lean_LocalContext_mkLocalDecl___spec__1(x_41, x_64, x_63); +x_66 = l_Lean_LocalDecl_index(x_63); +if (lean_is_scalar(x_62)) { + x_67 = lean_alloc_ctor(1, 1, 0); +} else { + x_67 = x_62; +} +lean_ctor_set(x_67, 0, x_63); +x_68 = l_Lean_PersistentArray_set___rarg(x_42, x_66, x_67); +lean_dec(x_66); +x_69 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_69, 0, x_65); +lean_ctor_set(x_69, 1, x_68); +lean_ctor_set(x_33, 0, x_69); +x_15 = x_33; +x_16 = x_39; +goto block_21; +} +} +} +else +{ +uint8_t x_70; +lean_free_object(x_33); +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_2); +lean_dec(x_1); +x_70 = !lean_is_exclusive(x_37); +if (x_70 == 0) +{ +return x_37; +} +else +{ +lean_object* x_71; lean_object* x_72; lean_object* x_73; +x_71 = lean_ctor_get(x_37, 0); +x_72 = lean_ctor_get(x_37, 1); +lean_inc(x_72); +lean_inc(x_71); +lean_dec(x_37); +x_73 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_73, 0, x_71); +lean_ctor_set(x_73, 1, x_72); +return x_73; +} +} +} +else +{ +lean_object* x_74; lean_object* x_75; lean_object* x_76; +x_74 = lean_ctor_get(x_33, 0); +lean_inc(x_74); +lean_dec(x_33); +lean_inc(x_1); +x_75 = lean_alloc_closure((void*)(l_Lean_Elab_Term_StructInst_DefaultFields_reduce), 7, 2); +lean_closure_set(x_75, 0, x_1); +lean_closure_set(x_75, 1, x_74); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_2); +lean_inc(x_6); +x_76 = l_Lean_Meta_withLCtx___at___private_Lean_Meta_Basic_0__Lean_Meta_mkLevelErrorMessageCore___spec__2___rarg(x_6, x_2, x_75, x_7, x_8, x_9, x_10, x_11); +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; +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_Expr_fvarId_x21(x_14); +lean_dec(x_14); +x_80 = lean_ctor_get(x_6, 0); +lean_inc(x_80); +x_81 = lean_ctor_get(x_6, 1); +lean_inc(x_81); +lean_inc(x_6); +x_82 = lean_local_ctx_find(x_6, x_79); +if (lean_obj_tag(x_82) == 0) +{ +lean_object* x_83; +lean_dec(x_81); +lean_dec(x_80); +lean_dec(x_77); +x_83 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_83, 0, x_6); +x_15 = x_83; +x_16 = x_78; +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; +if (lean_is_exclusive(x_6)) { + lean_ctor_release(x_6, 0); + lean_ctor_release(x_6, 1); + x_84 = x_6; +} else { + lean_dec_ref(x_6); + x_84 = lean_box(0); +} +x_85 = lean_ctor_get(x_82, 0); +lean_inc(x_85); +if (lean_is_exclusive(x_82)) { + lean_ctor_release(x_82, 0); + x_86 = x_82; +} else { + lean_dec_ref(x_82); + x_86 = lean_box(0); +} +x_87 = l_Lean_LocalDecl_setValue(x_85, x_77); +x_88 = l_Lean_LocalDecl_fvarId(x_87); +lean_inc(x_87); +x_89 = l_Lean_PersistentHashMap_insert___at_Lean_LocalContext_mkLocalDecl___spec__1(x_80, x_88, x_87); +x_90 = l_Lean_LocalDecl_index(x_87); +if (lean_is_scalar(x_86)) { + x_91 = lean_alloc_ctor(1, 1, 0); +} else { + x_91 = x_86; +} +lean_ctor_set(x_91, 0, x_87); +x_92 = l_Lean_PersistentArray_set___rarg(x_81, x_90, x_91); +lean_dec(x_90); +if (lean_is_scalar(x_84)) { + x_93 = lean_alloc_ctor(0, 2, 0); +} else { + x_93 = x_84; +} +lean_ctor_set(x_93, 0, x_89); +lean_ctor_set(x_93, 1, x_92); +x_94 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_94, 0, x_93); +x_15 = x_94; +x_16 = x_78; +goto block_21; +} +} +else +{ +lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; +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_2); +lean_dec(x_1); +x_95 = lean_ctor_get(x_76, 0); +lean_inc(x_95); +x_96 = lean_ctor_get(x_76, 1); +lean_inc(x_96); +if (lean_is_exclusive(x_76)) { + lean_ctor_release(x_76, 0); + lean_ctor_release(x_76, 1); + x_97 = x_76; +} else { + lean_dec_ref(x_76); + x_97 = lean_box(0); +} +if (lean_is_scalar(x_97)) { + x_98 = lean_alloc_ctor(1, 2, 0); +} else { + x_98 = x_97; +} +lean_ctor_set(x_98, 0, x_95); +lean_ctor_set(x_98, 1, x_96); +return x_98; +} +} +} +} +else +{ +lean_object* x_99; lean_object* x_100; +x_99 = lean_ctor_get(x_22, 0); +lean_inc(x_99); +lean_dec(x_22); +x_100 = l_Lean_LocalDecl_value_x3f(x_99); +lean_dec(x_99); +if (lean_obj_tag(x_100) == 0) +{ +lean_object* x_101; +lean_dec(x_14); +x_101 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_101, 0, x_6); +x_15 = x_101; +x_16 = x_11; +goto block_21; +} +else +{ +lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; +x_102 = lean_ctor_get(x_100, 0); +lean_inc(x_102); +if (lean_is_exclusive(x_100)) { + lean_ctor_release(x_100, 0); + x_103 = x_100; +} else { + lean_dec_ref(x_100); + x_103 = lean_box(0); +} +lean_inc(x_1); +x_104 = lean_alloc_closure((void*)(l_Lean_Elab_Term_StructInst_DefaultFields_reduce), 7, 2); +lean_closure_set(x_104, 0, x_1); +lean_closure_set(x_104, 1, x_102); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_2); +lean_inc(x_6); +x_105 = l_Lean_Meta_withLCtx___at___private_Lean_Meta_Basic_0__Lean_Meta_mkLevelErrorMessageCore___spec__2___rarg(x_6, x_2, x_104, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_105) == 0) +{ +lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; +x_106 = lean_ctor_get(x_105, 0); +lean_inc(x_106); +x_107 = lean_ctor_get(x_105, 1); +lean_inc(x_107); +lean_dec(x_105); +x_108 = l_Lean_Expr_fvarId_x21(x_14); +lean_dec(x_14); +x_109 = lean_ctor_get(x_6, 0); +lean_inc(x_109); +x_110 = lean_ctor_get(x_6, 1); +lean_inc(x_110); +lean_inc(x_6); +x_111 = lean_local_ctx_find(x_6, x_108); +if (lean_obj_tag(x_111) == 0) +{ +lean_object* x_112; +lean_dec(x_110); +lean_dec(x_109); +lean_dec(x_106); +if (lean_is_scalar(x_103)) { + x_112 = lean_alloc_ctor(1, 1, 0); +} else { + x_112 = x_103; +} +lean_ctor_set(x_112, 0, x_6); +x_15 = x_112; +x_16 = x_107; +goto block_21; +} +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; +if (lean_is_exclusive(x_6)) { + lean_ctor_release(x_6, 0); + lean_ctor_release(x_6, 1); + x_113 = x_6; +} else { + lean_dec_ref(x_6); + 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); +} +x_116 = l_Lean_LocalDecl_setValue(x_114, x_106); +x_117 = l_Lean_LocalDecl_fvarId(x_116); +lean_inc(x_116); +x_118 = l_Lean_PersistentHashMap_insert___at_Lean_LocalContext_mkLocalDecl___spec__1(x_109, x_117, x_116); +x_119 = l_Lean_LocalDecl_index(x_116); +if (lean_is_scalar(x_115)) { + x_120 = lean_alloc_ctor(1, 1, 0); +} else { + x_120 = x_115; +} +lean_ctor_set(x_120, 0, x_116); +x_121 = l_Lean_PersistentArray_set___rarg(x_110, x_119, x_120); +lean_dec(x_119); +if (lean_is_scalar(x_113)) { + x_122 = lean_alloc_ctor(0, 2, 0); +} else { + x_122 = x_113; +} +lean_ctor_set(x_122, 0, x_118); +lean_ctor_set(x_122, 1, x_121); +if (lean_is_scalar(x_103)) { + x_123 = lean_alloc_ctor(1, 1, 0); +} else { + x_123 = x_103; +} +lean_ctor_set(x_123, 0, x_122); +x_15 = x_123; +x_16 = x_107; +goto block_21; +} +} +else +{ +lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; +lean_dec(x_103); +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_2); +lean_dec(x_1); +x_124 = lean_ctor_get(x_105, 0); +lean_inc(x_124); +x_125 = lean_ctor_get(x_105, 1); +lean_inc(x_125); +if (lean_is_exclusive(x_105)) { + lean_ctor_release(x_105, 0); + lean_ctor_release(x_105, 1); + x_126 = x_105; +} else { + lean_dec_ref(x_105); + x_126 = lean_box(0); +} +if (lean_is_scalar(x_126)) { + x_127 = lean_alloc_ctor(1, 2, 0); +} else { + x_127 = x_126; +} +lean_ctor_set(x_127, 0, x_124); +lean_ctor_set(x_127, 1, x_125); +return x_127; +} +} +} +} +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_5, x_18); +x_5 = x_19; +x_6 = x_17; +x_11 = x_16; +goto _start; +} +} +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +uint8_t x_12; +x_12 = lean_usize_dec_lt(x_5, x_4); +if (x_12 == 0) +{ +lean_object* x_13; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_2); +lean_dec(x_1); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_6); +lean_ctor_set(x_13, 1, x_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_3, x_5); +lean_inc(x_6); +x_22 = l_Lean_LocalContext_findFVar_x3f(x_6, x_14); +if (lean_obj_tag(x_22) == 0) +{ +lean_object* x_23; lean_object* x_24; +lean_dec(x_14); +x_23 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___spec__3___closed__2; +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +x_24 = l_panic___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___spec__2(x_23, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_24) == 0) +{ +lean_object* x_25; lean_object* x_26; +x_25 = lean_ctor_get(x_24, 1); +lean_inc(x_25); +lean_dec(x_24); +x_26 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_26, 0, x_6); +x_15 = x_26; +x_16 = x_25; +goto block_21; +} +else +{ +uint8_t x_27; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_2); +lean_dec(x_1); +x_27 = !lean_is_exclusive(x_24); +if (x_27 == 0) +{ +return x_24; +} +else +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_24, 0); +x_29 = lean_ctor_get(x_24, 1); +lean_inc(x_29); +lean_inc(x_28); +lean_dec(x_24); +x_30 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +return x_30; +} +} +} +else +{ +uint8_t x_31; +x_31 = !lean_is_exclusive(x_22); +if (x_31 == 0) +{ +lean_object* x_32; lean_object* x_33; +x_32 = lean_ctor_get(x_22, 0); +x_33 = l_Lean_LocalDecl_value_x3f(x_32); +lean_dec(x_32); +if (lean_obj_tag(x_33) == 0) +{ +lean_dec(x_14); +lean_ctor_set(x_22, 0, x_6); +x_15 = x_22; +x_16 = x_11; +goto block_21; +} +else +{ +uint8_t x_34; +lean_free_object(x_22); +x_34 = !lean_is_exclusive(x_33); +if (x_34 == 0) +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_33, 0); +lean_inc(x_1); +x_36 = lean_alloc_closure((void*)(l_Lean_Elab_Term_StructInst_DefaultFields_reduce), 7, 2); +lean_closure_set(x_36, 0, x_1); +lean_closure_set(x_36, 1, x_35); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_2); +lean_inc(x_6); +x_37 = l_Lean_Meta_withLCtx___at___private_Lean_Meta_Basic_0__Lean_Meta_mkLevelErrorMessageCore___spec__2___rarg(x_6, x_2, x_36, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_37) == 0) +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; +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_fvarId_x21(x_14); +lean_dec(x_14); +x_41 = lean_ctor_get(x_6, 0); +lean_inc(x_41); +x_42 = lean_ctor_get(x_6, 1); +lean_inc(x_42); +lean_inc(x_6); +x_43 = lean_local_ctx_find(x_6, x_40); +if (lean_obj_tag(x_43) == 0) +{ +lean_dec(x_42); +lean_dec(x_41); +lean_dec(x_38); +lean_ctor_set(x_33, 0, x_6); +x_15 = x_33; +x_16 = x_39; +goto block_21; +} +else +{ +uint8_t x_44; +x_44 = !lean_is_exclusive(x_6); +if (x_44 == 0) +{ +lean_object* x_45; lean_object* x_46; uint8_t x_47; +x_45 = lean_ctor_get(x_6, 1); +lean_dec(x_45); +x_46 = lean_ctor_get(x_6, 0); +lean_dec(x_46); +x_47 = !lean_is_exclusive(x_43); +if (x_47 == 0) +{ +lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_48 = lean_ctor_get(x_43, 0); +x_49 = l_Lean_LocalDecl_setValue(x_48, x_38); +x_50 = l_Lean_LocalDecl_fvarId(x_49); +lean_inc(x_49); +x_51 = l_Lean_PersistentHashMap_insert___at_Lean_LocalContext_mkLocalDecl___spec__1(x_41, x_50, x_49); +x_52 = l_Lean_LocalDecl_index(x_49); +lean_ctor_set(x_43, 0, x_49); +x_53 = l_Lean_PersistentArray_set___rarg(x_42, x_52, x_43); +lean_dec(x_52); +lean_ctor_set(x_6, 1, x_53); +lean_ctor_set(x_6, 0, x_51); +lean_ctor_set(x_33, 0, x_6); +x_15 = x_33; +x_16 = x_39; +goto block_21; +} +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; +x_54 = lean_ctor_get(x_43, 0); +lean_inc(x_54); +lean_dec(x_43); +x_55 = l_Lean_LocalDecl_setValue(x_54, x_38); +x_56 = l_Lean_LocalDecl_fvarId(x_55); +lean_inc(x_55); +x_57 = l_Lean_PersistentHashMap_insert___at_Lean_LocalContext_mkLocalDecl___spec__1(x_41, x_56, x_55); +x_58 = l_Lean_LocalDecl_index(x_55); +x_59 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_59, 0, x_55); +x_60 = l_Lean_PersistentArray_set___rarg(x_42, x_58, x_59); +lean_dec(x_58); +lean_ctor_set(x_6, 1, x_60); +lean_ctor_set(x_6, 0, x_57); +lean_ctor_set(x_33, 0, x_6); +x_15 = x_33; +x_16 = x_39; +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_dec(x_6); +x_61 = lean_ctor_get(x_43, 0); +lean_inc(x_61); +if (lean_is_exclusive(x_43)) { + lean_ctor_release(x_43, 0); + x_62 = x_43; +} else { + lean_dec_ref(x_43); + x_62 = lean_box(0); +} +x_63 = l_Lean_LocalDecl_setValue(x_61, x_38); +x_64 = l_Lean_LocalDecl_fvarId(x_63); +lean_inc(x_63); +x_65 = l_Lean_PersistentHashMap_insert___at_Lean_LocalContext_mkLocalDecl___spec__1(x_41, x_64, x_63); +x_66 = l_Lean_LocalDecl_index(x_63); +if (lean_is_scalar(x_62)) { + x_67 = lean_alloc_ctor(1, 1, 0); +} else { + x_67 = x_62; +} +lean_ctor_set(x_67, 0, x_63); +x_68 = l_Lean_PersistentArray_set___rarg(x_42, x_66, x_67); +lean_dec(x_66); +x_69 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_69, 0, x_65); +lean_ctor_set(x_69, 1, x_68); +lean_ctor_set(x_33, 0, x_69); +x_15 = x_33; +x_16 = x_39; +goto block_21; +} +} +} +else +{ +uint8_t x_70; +lean_free_object(x_33); +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_2); +lean_dec(x_1); +x_70 = !lean_is_exclusive(x_37); +if (x_70 == 0) +{ +return x_37; +} +else +{ +lean_object* x_71; lean_object* x_72; lean_object* x_73; +x_71 = lean_ctor_get(x_37, 0); +x_72 = lean_ctor_get(x_37, 1); +lean_inc(x_72); +lean_inc(x_71); +lean_dec(x_37); +x_73 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_73, 0, x_71); +lean_ctor_set(x_73, 1, x_72); +return x_73; +} +} +} +else +{ +lean_object* x_74; lean_object* x_75; lean_object* x_76; +x_74 = lean_ctor_get(x_33, 0); +lean_inc(x_74); +lean_dec(x_33); +lean_inc(x_1); +x_75 = lean_alloc_closure((void*)(l_Lean_Elab_Term_StructInst_DefaultFields_reduce), 7, 2); +lean_closure_set(x_75, 0, x_1); +lean_closure_set(x_75, 1, x_74); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_2); +lean_inc(x_6); +x_76 = l_Lean_Meta_withLCtx___at___private_Lean_Meta_Basic_0__Lean_Meta_mkLevelErrorMessageCore___spec__2___rarg(x_6, x_2, x_75, x_7, x_8, x_9, x_10, x_11); +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; +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_Expr_fvarId_x21(x_14); +lean_dec(x_14); +x_80 = lean_ctor_get(x_6, 0); +lean_inc(x_80); +x_81 = lean_ctor_get(x_6, 1); +lean_inc(x_81); +lean_inc(x_6); +x_82 = lean_local_ctx_find(x_6, x_79); +if (lean_obj_tag(x_82) == 0) +{ +lean_object* x_83; +lean_dec(x_81); +lean_dec(x_80); +lean_dec(x_77); +x_83 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_83, 0, x_6); +x_15 = x_83; +x_16 = x_78; +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; +if (lean_is_exclusive(x_6)) { + lean_ctor_release(x_6, 0); + lean_ctor_release(x_6, 1); + x_84 = x_6; +} else { + lean_dec_ref(x_6); + x_84 = lean_box(0); +} +x_85 = lean_ctor_get(x_82, 0); +lean_inc(x_85); +if (lean_is_exclusive(x_82)) { + lean_ctor_release(x_82, 0); + x_86 = x_82; +} else { + lean_dec_ref(x_82); + x_86 = lean_box(0); +} +x_87 = l_Lean_LocalDecl_setValue(x_85, x_77); +x_88 = l_Lean_LocalDecl_fvarId(x_87); +lean_inc(x_87); +x_89 = l_Lean_PersistentHashMap_insert___at_Lean_LocalContext_mkLocalDecl___spec__1(x_80, x_88, x_87); +x_90 = l_Lean_LocalDecl_index(x_87); +if (lean_is_scalar(x_86)) { + x_91 = lean_alloc_ctor(1, 1, 0); +} else { + x_91 = x_86; +} +lean_ctor_set(x_91, 0, x_87); +x_92 = l_Lean_PersistentArray_set___rarg(x_81, x_90, x_91); +lean_dec(x_90); +if (lean_is_scalar(x_84)) { + x_93 = lean_alloc_ctor(0, 2, 0); +} else { + x_93 = x_84; +} +lean_ctor_set(x_93, 0, x_89); +lean_ctor_set(x_93, 1, x_92); +x_94 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_94, 0, x_93); +x_15 = x_94; +x_16 = x_78; +goto block_21; +} +} +else +{ +lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; +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_2); +lean_dec(x_1); +x_95 = lean_ctor_get(x_76, 0); +lean_inc(x_95); +x_96 = lean_ctor_get(x_76, 1); +lean_inc(x_96); +if (lean_is_exclusive(x_76)) { + lean_ctor_release(x_76, 0); + lean_ctor_release(x_76, 1); + x_97 = x_76; +} else { + lean_dec_ref(x_76); + x_97 = lean_box(0); +} +if (lean_is_scalar(x_97)) { + x_98 = lean_alloc_ctor(1, 2, 0); +} else { + x_98 = x_97; +} +lean_ctor_set(x_98, 0, x_95); +lean_ctor_set(x_98, 1, x_96); +return x_98; +} +} +} +} +else +{ +lean_object* x_99; lean_object* x_100; +x_99 = lean_ctor_get(x_22, 0); +lean_inc(x_99); +lean_dec(x_22); +x_100 = l_Lean_LocalDecl_value_x3f(x_99); +lean_dec(x_99); +if (lean_obj_tag(x_100) == 0) +{ +lean_object* x_101; +lean_dec(x_14); +x_101 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_101, 0, x_6); +x_15 = x_101; +x_16 = x_11; +goto block_21; +} +else +{ +lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; +x_102 = lean_ctor_get(x_100, 0); +lean_inc(x_102); +if (lean_is_exclusive(x_100)) { + lean_ctor_release(x_100, 0); + x_103 = x_100; +} else { + lean_dec_ref(x_100); + x_103 = lean_box(0); +} +lean_inc(x_1); +x_104 = lean_alloc_closure((void*)(l_Lean_Elab_Term_StructInst_DefaultFields_reduce), 7, 2); +lean_closure_set(x_104, 0, x_1); +lean_closure_set(x_104, 1, x_102); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_2); +lean_inc(x_6); +x_105 = l_Lean_Meta_withLCtx___at___private_Lean_Meta_Basic_0__Lean_Meta_mkLevelErrorMessageCore___spec__2___rarg(x_6, x_2, x_104, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_105) == 0) +{ +lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; +x_106 = lean_ctor_get(x_105, 0); +lean_inc(x_106); +x_107 = lean_ctor_get(x_105, 1); +lean_inc(x_107); +lean_dec(x_105); +x_108 = l_Lean_Expr_fvarId_x21(x_14); +lean_dec(x_14); +x_109 = lean_ctor_get(x_6, 0); +lean_inc(x_109); +x_110 = lean_ctor_get(x_6, 1); +lean_inc(x_110); +lean_inc(x_6); +x_111 = lean_local_ctx_find(x_6, x_108); +if (lean_obj_tag(x_111) == 0) +{ +lean_object* x_112; +lean_dec(x_110); +lean_dec(x_109); +lean_dec(x_106); +if (lean_is_scalar(x_103)) { + x_112 = lean_alloc_ctor(1, 1, 0); +} else { + x_112 = x_103; +} +lean_ctor_set(x_112, 0, x_6); +x_15 = x_112; +x_16 = x_107; +goto block_21; +} +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; +if (lean_is_exclusive(x_6)) { + lean_ctor_release(x_6, 0); + lean_ctor_release(x_6, 1); + x_113 = x_6; +} else { + lean_dec_ref(x_6); + 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); +} +x_116 = l_Lean_LocalDecl_setValue(x_114, x_106); +x_117 = l_Lean_LocalDecl_fvarId(x_116); +lean_inc(x_116); +x_118 = l_Lean_PersistentHashMap_insert___at_Lean_LocalContext_mkLocalDecl___spec__1(x_109, x_117, x_116); +x_119 = l_Lean_LocalDecl_index(x_116); +if (lean_is_scalar(x_115)) { + x_120 = lean_alloc_ctor(1, 1, 0); +} else { + x_120 = x_115; +} +lean_ctor_set(x_120, 0, x_116); +x_121 = l_Lean_PersistentArray_set___rarg(x_110, x_119, x_120); +lean_dec(x_119); +if (lean_is_scalar(x_113)) { + x_122 = lean_alloc_ctor(0, 2, 0); +} else { + x_122 = x_113; +} +lean_ctor_set(x_122, 0, x_118); +lean_ctor_set(x_122, 1, x_121); +if (lean_is_scalar(x_103)) { + x_123 = lean_alloc_ctor(1, 1, 0); +} else { + x_123 = x_103; +} +lean_ctor_set(x_123, 0, x_122); +x_15 = x_123; +x_16 = x_107; +goto block_21; +} +} +else +{ +lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; +lean_dec(x_103); +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_2); +lean_dec(x_1); +x_124 = lean_ctor_get(x_105, 0); +lean_inc(x_124); +x_125 = lean_ctor_get(x_105, 1); +lean_inc(x_125); +if (lean_is_exclusive(x_105)) { + lean_ctor_release(x_105, 0); + lean_ctor_release(x_105, 1); + x_126 = x_105; +} else { + lean_dec_ref(x_105); + x_126 = lean_box(0); +} +if (lean_is_scalar(x_126)) { + x_127 = lean_alloc_ctor(1, 2, 0); +} else { + x_127 = x_126; +} +lean_ctor_set(x_127, 0, x_124); +lean_ctor_set(x_127, 1, x_125); +return x_127; +} +} +} +} +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_5, x_18); +x_5 = x_19; +x_6 = x_17; +x_11 = x_16; +goto _start; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_reduce___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; size_t x_13; size_t x_14; lean_object* x_15; +x_9 = l_Lean_Meta_getLocalInstances(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 = 0; -x_13 = 1; -x_14 = 1; -x_15 = l_Lean_Meta_mkLambdaFVars(x_2, x_10, x_12, x_13, x_12, x_14, x_4, x_5, x_6, x_7, x_11); +x_12 = lean_ctor_get(x_4, 1); +lean_inc(x_12); +x_13 = lean_array_size(x_2); +x_14 = 0; +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_10); +lean_inc(x_1); +x_15 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___spec__3(x_1, x_10, x_2, x_13, x_14, x_12, x_4, x_5, x_6, x_7, x_11); +if (lean_obj_tag(x_15) == 0) +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_15, 1); +lean_inc(x_17); +lean_dec(x_15); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_18 = l_Lean_Elab_Term_StructInst_DefaultFields_reduce(x_1, x_3, x_4, x_5, x_6, x_7, x_17); +if (lean_obj_tag(x_18) == 0) +{ +lean_object* x_19; lean_object* x_20; uint8_t x_21; uint8_t x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +x_20 = lean_ctor_get(x_18, 1); +lean_inc(x_20); +lean_dec(x_18); +x_21 = 1; +x_22 = 1; +x_23 = lean_box(x_21); +x_24 = lean_box(x_22); +x_25 = lean_alloc_closure((void*)(l_Lean_Meta_mkLetFVars___boxed), 9, 4); +lean_closure_set(x_25, 0, x_2); +lean_closure_set(x_25, 1, x_19); +lean_closure_set(x_25, 2, x_23); +lean_closure_set(x_25, 3, x_24); +x_26 = l_Lean_Meta_withLCtx___at___private_Lean_Meta_Basic_0__Lean_Meta_mkLevelErrorMessageCore___spec__2___rarg(x_16, x_10, x_25, x_4, x_5, x_6, x_7, x_20); +return x_26; +} +else +{ +uint8_t x_27; +lean_dec(x_16); +lean_dec(x_10); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -return x_15; +lean_dec(x_2); +x_27 = !lean_is_exclusive(x_18); +if (x_27 == 0) +{ +return x_18; } else { -uint8_t x_16; +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_18, 0); +x_29 = lean_ctor_get(x_18, 1); +lean_inc(x_29); +lean_inc(x_28); +lean_dec(x_18); +x_30 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +return x_30; +} +} +} +else +{ +uint8_t x_31; +lean_dec(x_10); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); -x_16 = !lean_is_exclusive(x_9); -if (x_16 == 0) +lean_dec(x_1); +x_31 = !lean_is_exclusive(x_15); +if (x_31 == 0) { -return x_9; +return x_15; } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_9, 0); -x_18 = lean_ctor_get(x_9, 1); -lean_inc(x_18); -lean_inc(x_17); -lean_dec(x_9); -x_19 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_19, 0, x_17); -lean_ctor_set(x_19, 1, x_18); -return x_19; +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_15, 0); +x_33 = lean_ctor_get(x_15, 1); +lean_inc(x_33); +lean_inc(x_32); +lean_dec(x_15); +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; } } } @@ -30237,6 +31490,122 @@ return x_19; } } } +LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_reduce___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; lean_object* x_10; lean_object* x_11; lean_object* x_12; size_t x_13; size_t x_14; lean_object* x_15; +x_9 = l_Lean_Meta_getLocalInstances(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_ctor_get(x_4, 1); +lean_inc(x_12); +x_13 = lean_array_size(x_2); +x_14 = 0; +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_10); +lean_inc(x_1); +x_15 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___spec__4(x_1, x_10, x_2, x_13, x_14, x_12, x_4, x_5, x_6, x_7, x_11); +if (lean_obj_tag(x_15) == 0) +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_15, 1); +lean_inc(x_17); +lean_dec(x_15); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_18 = l_Lean_Elab_Term_StructInst_DefaultFields_reduce(x_1, x_3, x_4, x_5, x_6, x_7, x_17); +if (lean_obj_tag(x_18) == 0) +{ +lean_object* x_19; lean_object* x_20; uint8_t x_21; uint8_t x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +x_20 = lean_ctor_get(x_18, 1); +lean_inc(x_20); +lean_dec(x_18); +x_21 = 1; +x_22 = 1; +x_23 = lean_box(x_21); +x_24 = lean_box(x_22); +x_25 = lean_alloc_closure((void*)(l_Lean_Meta_mkLetFVars___boxed), 9, 4); +lean_closure_set(x_25, 0, x_2); +lean_closure_set(x_25, 1, x_19); +lean_closure_set(x_25, 2, x_23); +lean_closure_set(x_25, 3, x_24); +x_26 = l_Lean_Meta_withLCtx___at___private_Lean_Meta_Basic_0__Lean_Meta_mkLevelErrorMessageCore___spec__2___rarg(x_16, x_10, x_25, x_4, x_5, x_6, x_7, x_20); +return x_26; +} +else +{ +uint8_t x_27; +lean_dec(x_16); +lean_dec(x_10); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +x_27 = !lean_is_exclusive(x_18); +if (x_27 == 0) +{ +return x_18; +} +else +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_18, 0); +x_29 = lean_ctor_get(x_18, 1); +lean_inc(x_29); +lean_inc(x_28); +lean_dec(x_18); +x_30 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +return x_30; +} +} +} +else +{ +uint8_t x_31; +lean_dec(x_10); +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_31 = !lean_is_exclusive(x_15); +if (x_31 == 0) +{ +return x_15; +} +else +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_15, 0); +x_33 = lean_ctor_get(x_15, 1); +lean_inc(x_33); +lean_inc(x_32); +lean_dec(x_15); +x_34 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_34, 0, x_32); +lean_ctor_set(x_34, 1, x_33); +return x_34; +} +} +} +} static lean_object* _init_l_Lean_Elab_Term_StructInst_DefaultFields_reduce___closed__1() { _start: { @@ -30359,7 +31728,7 @@ lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; uint8_t x x_26 = lean_ctor_get(x_2, 0); lean_inc(x_26); lean_inc(x_1); -x_27 = lean_alloc_closure((void*)(l_Array_contains___at_Lean_findField_x3f___spec__1___boxed), 2, 1); +x_27 = lean_alloc_closure((void*)(l_Array_contains___at_Lean_registerInternalExceptionId___spec__1___boxed), 2, 1); lean_closure_set(x_27, 0, x_1); x_28 = lean_ctor_get(x_3, 0); lean_inc(x_28); @@ -30625,7 +31994,7 @@ return x_103; case 8: { lean_object* x_104; uint8_t x_105; lean_object* x_106; -x_104 = lean_alloc_closure((void*)(l_Lean_Elab_Term_StructInst_DefaultFields_reduce___lambda__1), 8, 1); +x_104 = lean_alloc_closure((void*)(l_Lean_Elab_Term_StructInst_DefaultFields_reduce___lambda__3), 8, 1); lean_closure_set(x_104, 0, x_1); x_105 = 0; x_106 = l_Lean_Meta_lambdaLetTelescope___at___private_Lean_Meta_InferType_0__Lean_Meta_inferLambdaType___spec__1___rarg(x_2, x_104, x_105, x_3, x_4, x_5, x_6, x_7); @@ -31016,6 +32385,32 @@ x_12 = l_Array_mapMUnsafe_map___at_Lean_Elab_Term_StructInst_DefaultFields_reduc return x_12; } } +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___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; +x_12 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_13 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_14 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___spec__3(x_1, x_2, x_3, x_12, x_13, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_3); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___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) { +_start: +{ +size_t x_12; size_t x_13; lean_object* x_14; +x_12 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_13 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_14 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___spec__4(x_1, x_2, x_3, x_12, x_13, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_3); +return x_14; +} +} LEAN_EXPORT uint8_t l_Lean_Elab_Term_StructInst_DefaultFields_tryToSynthesizeDefault_loop___lambda__1(lean_object* x_1) { _start: { @@ -31876,7 +33271,7 @@ static lean_object* _init_l_List_forIn_loop___at_Lean_Elab_Term_StructInst_Defau lean_object* x_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___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_getStructSource___spec__2___closed__1; x_2 = l_List_forIn_loop___at_Lean_Elab_Term_StructInst_DefaultFields_step___spec__3___closed__1; -x_3 = lean_unsigned_to_nat(895u); +x_3 = lean_unsigned_to_nat(908u); x_4 = lean_unsigned_to_nat(25u); x_5 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_getStructSource___spec__2___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -37115,7 +38510,7 @@ x_4 = l_Lean_addBuiltinDeclarationRanges(x_2, x_3, x_1); return x_4; } } -static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__1() { +static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -37125,37 +38520,37 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__2() { +static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__1; +x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__1; x_2 = l___regBuiltin_Lean_Elab_Term_StructInst_expandStructInstExpectedType__1___closed__3; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__3() { +static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__2; +x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__2; x_2 = l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__7; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__4() { +static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__3; +x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__3; x_2 = l___regBuiltin_Lean_Elab_Term_StructInst_expandStructInstExpectedType__1___closed__4; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__5() { +static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__5() { _start: { lean_object* x_1; @@ -37163,17 +38558,17 @@ x_1 = lean_mk_string_unchecked("initFn", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__6() { +static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__4; -x_2 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__5; +x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__4; +x_2 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__5; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__7() { +static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__7() { _start: { lean_object* x_1; @@ -37181,47 +38576,47 @@ x_1 = lean_mk_string_unchecked("_@", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__8() { +static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__6; -x_2 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__7; +x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__6; +x_2 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__7; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__9() { +static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__8; +x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__8; x_2 = l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__5; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__10() { +static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__9; +x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__9; x_2 = l___regBuiltin_Lean_Elab_Term_StructInst_expandStructInstExpectedType__1___closed__3; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__11() { +static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__10; +x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__10; x_2 = l___regBuiltin_Lean_Elab_Term_StructInst_expandStructInstExpectedType__1___closed__4; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__12() { +static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__12() { _start: { lean_object* x_1; @@ -37229,33 +38624,33 @@ x_1 = lean_mk_string_unchecked("_hyg", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__13() { +static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__11; -x_2 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__12; +x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__11; +x_2 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__12; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__14() { +static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__13; -x_2 = lean_unsigned_to_nat(13312u); +x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__13; +x_2 = lean_unsigned_to_nat(13688u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688_(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; x_2 = l_List_foldlM___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStruct___spec__5___closed__3; x_3 = 0; -x_4 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__14; +x_4 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__14; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); if (lean_obj_tag(x_5) == 0) { @@ -37827,6 +39222,12 @@ l_Lean_Elab_Term_StructInst_DefaultFields_mkDefaultValueAux_x3f___closed__4 = _i lean_mark_persistent(l_Lean_Elab_Term_StructInst_DefaultFields_mkDefaultValueAux_x3f___closed__4); l_Lean_Elab_Term_StructInst_DefaultFields_mkDefaultValueAux_x3f___closed__5 = _init_l_Lean_Elab_Term_StructInst_DefaultFields_mkDefaultValueAux_x3f___closed__5(); lean_mark_persistent(l_Lean_Elab_Term_StructInst_DefaultFields_mkDefaultValueAux_x3f___closed__5); +l_panic___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___spec__2___closed__1 = _init_l_panic___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___spec__2___closed__1(); +lean_mark_persistent(l_panic___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___spec__2___closed__1); +l_Array_forInUnsafe_loop___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___spec__3___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___spec__3___closed__1(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___spec__3___closed__1); +l_Array_forInUnsafe_loop___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___spec__3___closed__2 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___spec__3___closed__2(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Term_StructInst_DefaultFields_reduce___spec__3___closed__2); l_Lean_Elab_Term_StructInst_DefaultFields_reduce___closed__1 = _init_l_Lean_Elab_Term_StructInst_DefaultFields_reduce___closed__1(); lean_mark_persistent(l_Lean_Elab_Term_StructInst_DefaultFields_reduce___closed__1); l_Lean_Elab_Term_StructInst_DefaultFields_tryToSynthesizeDefault_loop___closed__1 = _init_l_Lean_Elab_Term_StructInst_DefaultFields_tryToSynthesizeDefault_loop___closed__1(); @@ -37916,35 +39317,35 @@ lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_StructInst_elabStructInst_dec if (builtin) {res = l___regBuiltin_Lean_Elab_Term_StructInst_elabStructInst_declRange__1(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__1 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__1(); -lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__1); -l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__2 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__2(); -lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__2); -l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__3 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__3(); -lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__3); -l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__4 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__4(); -lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__4); -l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__5 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__5(); -lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__5); -l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__6 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__6(); -lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__6); -l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__7 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__7(); -lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__7); -l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__8 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__8(); -lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__8); -l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__9 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__9(); -lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__9); -l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__10 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__10(); -lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__10); -l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__11 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__11(); -lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__11); -l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__12 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__12(); -lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__12); -l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__13 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__13(); -lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__13); -l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__14 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__14(); -lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__14); -if (builtin) {res = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312_(lean_io_mk_world()); +}l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__1 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__1(); +lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__1); +l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__2 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__2(); +lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__2); +l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__3 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__3(); +lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__3); +l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__4 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__4(); +lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__4); +l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__5 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__5(); +lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__5); +l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__6 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__6(); +lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__6); +l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__7 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__7(); +lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__7); +l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__8 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__8(); +lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__8); +l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__9 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__9(); +lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__9); +l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__10 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__10(); +lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__10); +l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__11 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__11(); +lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__11); +l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__12 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__12(); +lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__12); +l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__13 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__13(); +lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__13); +l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__14 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__14(); +lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688____closed__14); +if (builtin) {res = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13688_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }return lean_io_result_mk_ok(lean_box(0)); diff --git a/stage0/stdlib/Lean/Elab/Structure.c b/stage0/stdlib/Lean/Elab/Structure.c index 2d79f61f3af5..b019e0f935a0 100644 --- a/stage0/stdlib/Lean/Elab/Structure.c +++ b/stage0/stdlib/Lean/Elab/Structure.c @@ -14,135 +14,125 @@ extern "C" { #endif static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___closed__5; -LEAN_EXPORT lean_object* l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__5(lean_object*, size_t, size_t, lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___lambda__1___boxed(lean_object*); lean_object* l_Lean_setReducibilityStatus___at___private_Lean_Meta_Constructions_BRecOn_0__Lean_mkBelowFromRec___spec__7(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_string_utf8_extract(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*); 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_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_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___lambda__9(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__21; 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*); -static lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___closed__1; +lean_object* l_Lean_Elab_Term_withoutSavingRecAppSyntax___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_reprPrec(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__7; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___lambda__10(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 uint8_t l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabFieldTypeValue___lambda__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_structureSyntaxToView___closed__2; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent_copyFields___spec__2___closed__1; -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__22; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__2; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withStructureLocalDecl___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_toVisibility___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__4___boxed(lean_object**); lean_object* l_Option_repr___at___private_Lean_Meta_Transform_0__Lean_reprTransformStep____x40_Lean_Meta_Transform___hyg_45____spec__1(lean_object*, lean_object*); +static lean_object* l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__2; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions(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__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___lambda__1(lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__8; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType(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_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481_(uint8_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUsed___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_checkValidFieldModifier___closed__2; -lean_object* l_Lean_MapDeclarationExtension_insert___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__8; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___lambda__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructureView___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_Command_instDecidableEqStructFieldKind___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_StructFieldKind_toCtorIdx___boxed(lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__4; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__6; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields___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_expandFields___closed__11; LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___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_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__3___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); lean_object* l_Lean_mkAppN(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__1___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_collectLevelParamsInFVar___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___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___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_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___spec__2___closed__2; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields_go___spec__2___closed__5; -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__3; -static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__9; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__22; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom___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_liftMacroM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__5___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_processOveriddenDefaultValues___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__9___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_Structure_0__Lean_Elab_Command_elabStructureView___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* l_Lean_Meta_mkFreshLevelMVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__3; lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); lean_object* l_Lean_NameSet_contains___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_replaceFieldInfo___spec__1(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabStructureViewPostprocessing___spec__1(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkSizeOfInstances(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__8(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_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__15; lean_object* l_Lean_Elab_Command_checkResultingUniverse(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_getProjectionFnInfo_x3f___at_Lean_Meta_getStuckMVar_x3f___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent(lean_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_mkCoercionToCopiedParent(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Command_runTermElabM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_sortDeclLevelParams(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_throwError___at___private_Lean_Elab_Command_0__Lean_Elab_Command_elabCommandUsing___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__11___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -extern lean_object* l_Lean_declRangeExt; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__11; +lean_object* l_Lean_Elab_Command_checkValidInductiveModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1(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__5___closed__1; lean_object* l_Lean_Elab_Command_mkResultUniverse(lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___spec__1(lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___lambda__1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__6; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__1___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__1; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___closed__3; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__6; lean_object* l_Lean_ConstantInfo_type(lean_object*); lean_object* lean_whnf(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___boxed(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_Structure_0__Lean_Elab_Command_elabParents_go___rarg___lambda__1(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__6; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__13; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidFieldModifier___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -extern lean_object* l_Lean_maxRecDepthErrorMessage; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__5___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_Structure_0__Lean_Elab_Command_expandCtor___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_Elab_Command_elabStructure___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateFieldInfoVal___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_indentD(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectLevelParamsInFVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__10; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectLevelParamsInFVars___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -uint8_t l_Lean_Exception_isInterrupt(lean_object*); -static lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__1; -lean_object* l_Lean_Elab_Command_getMainModule___rarg(lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_synthesizeSyntheticMVars(uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___closed__4; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__25; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__7; +static lean_object* l_Lean_Elab_Command_elabStructure___lambda__2___closed__1; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__10; lean_object* l_Lean_Meta_isExprDefEq(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_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_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_validStructType___boxed(lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__23; -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__4; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___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_Elab_Structure_0__Lean_Elab_Command_setSourceInstImplicit___closed__1; -static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__7; lean_object* l_Lean_Level_addOffsetAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectLevelParamsInStructure___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_getAutoParamTactic_x3f(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUsed___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isAppOfArity(lean_object*, lean_object*, lean_object*); -LEAN_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_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__9; +static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__16; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__6; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent_copyFields(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__14; +static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__13; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__5; +static lean_object* l_Lean_Elab_Command_instInhabitedStructParentInfo___closed__2; lean_object* l_Lean_findDocString_x3f(lean_object*, lean_object*, uint8_t, lean_object*); -static lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___lambda__3___boxed(lean_object**); lean_object* l_Lean_Name_toString(lean_object*, uint8_t, lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__15; LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__6(lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__13; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022_(lean_object*); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__4; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4___closed__1; lean_object* l_Lean_Syntax_getId(lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__19; @@ -152,30 +142,32 @@ static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandC 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*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_sort___override(lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__3; +lean_object* l_Lean_MessageData_ofList(lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__7; uint8_t lean_nat_dec_le(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__9___rarg___closed__2; lean_object* lean_array_push(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__7(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__1; lean_object* l_Array_toSubarray___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_setSourceInstImplicit(lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwKernelException___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___closed__5; -static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__5; -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__26; -uint8_t l_Array_contains___at_Lean_findField_x3f___spec__1(lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__11; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_mkStructureDecl___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_forM___at_Lean_Elab_Command_mkStructureDecl___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkFreshId___at_Lean_Meta_mkFreshExprMVarAt___spec__2___rarg(lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__15; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_go_x3f___closed__1; lean_object* lean_mk_array(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields_go___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___lambda__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_eq(size_t, size_t); -static lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__4; lean_object* l_Lean_Syntax_getArgs(lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__3; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instReprStructFieldInfo___closed__1; lean_object* l_Lean_replaceRef(lean_object*, lean_object*); static uint8_t l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__3; @@ -183,205 +175,191 @@ lean_object* l_Lean_throwError___at_Lean_Elab_Term_throwErrorIfErrors___spec__1( LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidFieldModifier(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_Command_StructFieldInfo_isFromParent(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_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__17; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___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_Syntax_getPos_x3f(lean_object*, uint8_t); lean_object* l_Lean_Expr_bvar___override(lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___lambda__1(lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectLevelParamsInStructure___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_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__5; -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_elabStructure___closed__2; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__9; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__1; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__1; -lean_object* l_Lean_Syntax_getTailPos_x3f(lean_object*, uint8_t); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__20; -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__3; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkInductiveType(lean_object*, lean_object*, lean_object*, 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_Structure_0__Lean_Elab_Command_containsFieldName(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__13; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4___boxed(lean_object**); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCtor(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__10(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_elabStructureView___closed__1; -static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__4___closed__1; lean_object* l_Lean_Expr_fvarId_x21(lean_object*); -lean_object* l_Lean_Elab_logException___at_Lean_Elab_Term_exceptionToSorry___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_structureDiamondWarning; -static lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__5; -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__11___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_elabParents___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__4; lean_object* lean_environment_find(lean_object*, lean_object*); +static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__11; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_toVisibility___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParamFVars___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___closed__1; static lean_object* l_Lean_Elab_Command_checkValidFieldModifier___lambda__1___closed__2; lean_object* l_Lean_Elab_Term_declareTacticSyntax(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_RBNode_insert___at_Lean_NameSet_insert___spec__1(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__1___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__15; -LEAN_EXPORT lean_object* l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__4; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__4; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__10; static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkIdentFrom(lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__3(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_instInhabitedStructCtorView___closed__2; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___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_Elab_addAuxDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__18___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateFieldInfoVal___spec__1(lean_object*, lean_object*, size_t, size_t, lean_object*); -uint8_t l_Lean_Linter_getLinterValue(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__5___lambda__3(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; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getResultUniverse___closed__2; +static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__10; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___closed__2; -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___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_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__13; lean_object* l_Lean_Syntax_node5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__5___boxed(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_updateResultingUniverse___lambda__2___closed__2; +size_t lean_usize_of_nat(lean_object*); lean_object* l_Nat_nextPowerOfTwo_go(lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_IndPredBelow_mkBelow(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_elabStructHeader___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_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Command_instInhabitedStructFieldInfo; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___closed__3; lean_object* l_Lean_stringToMessageData(lean_object*); -static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__8; -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__20; -LEAN_EXPORT lean_object* l_Lean_Elab_elabDeclAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__6; -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParamFVars___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*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_StructFieldInfo_isSubobject___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_processOveriddenDefaultValues(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -uint8_t l_Lean_MapDeclarationExtension_contains___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___closed__1; -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_mkSynthetic(lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___lambda__3___boxed(lean_object**); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__23; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_go_x3f(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___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__2___boxed(lean_object**); lean_object* l_Lean_Elab_Term_instInhabitedTermElabM(lean_object*); -static lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___spec__2___closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withStructureLocalDecl(lean_object*); static lean_object* l_Lean_Elab_Command_checkValidFieldModifier___lambda__1___closed__1; -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_structureSyntaxToView___spec__1___closed__2; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___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*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__3; -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___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_string_utf8_byte_size(lean_object*); +static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__6; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f___spec__1(lean_object*, lean_object*, lean_object*, size_t, size_t, 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_698____closed__16; lean_object* l_Lean_CollectLevelParams_main(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__9(lean_object*); -static lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__3___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__19___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___boxed__const__1; lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Meta_GeneralizeTelescope_generalizeTelescopeAux___spec__1___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_appArg_x21(lean_object*); -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*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_isPropCandidate___boxed(lean_object*); -LEAN_EXPORT 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___private_Lean_Elab_Structure_0__Lean_Elab_Command_levelMVarToParam___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__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructureViewPostprocessing___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__6; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__5; lean_object* l_Lean_mkDefaultFnOfProjFn(lean_object*); lean_object* l_List_mapTR_loop___at_Lean_mkConstWithLevelParams___spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__16; -static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__11___closed__2; +lean_object* l_Lean_LocalDecl_index(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_withSaveInfoContext___at___private_Lean_Elab_PreDefinition_Basic_0__Lean_Elab_addNonRecAux___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_getStructureFields(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateFieldInfoVal___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__9___rarg(lean_object*); +static lean_object* l_Lean_Elab_Command_mkStructureDecl___lambda__8___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom___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 uint8_t l_Lean_Elab_Command_instDecidableEqStructFieldKind(uint8_t, uint8_t); +static lean_object* l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__4; lean_object* l_Lean_getDefaultFnForField_x3f(lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__8; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkInductiveType___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_elabTermEnsuringType___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___closed__3; -static lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__2___closed__1; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__7; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__4; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__21; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields_go___spec__2___closed__9; -static lean_object* l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__3; +static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__14; +lean_object* l_Lean_PersistentArray_set___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_panic___at___private_Lean_Meta_InferType_0__Lean_Meta_checkInferTypeCache___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___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*, lean_object*); size_t lean_ptr_addr(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8(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_Structure_0__Lean_Elab_Command_isPropCandidate(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__25; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__2___closed__2; lean_object* l_Lean_Elab_Modifiers_addAttr(lean_object*, lean_object*); +lean_object* l___private_Init_Meta_0__Lean_Syntax_reprSyntax____x40_Init_Meta___hyg_2168_(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*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader(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__2___closed__1; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339_(uint8_t, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__4; +static lean_object* l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__5; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields_go___spec__2___closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__9___rarg___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___lambda__7___boxed(lean_object**); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__14; size_t lean_usize_of_nat(lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_TagDeclarationExtension_isTagged(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectLevelParamsInFVars___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__1; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__22; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_removeUnused___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getResultUniverse___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParamFVars(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__2; lean_object* lean_expr_abstract(lean_object*, lean_object*); lean_object* l_Lean_Meta_withLCtx___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go(lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__20; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__6; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__7___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_StructFieldKind_noConfusion___rarg___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__22; LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidFieldModifier___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidFieldModifier___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___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT uint8_t l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields_go___spec__2(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__1; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__4; -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__9; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabFieldTypeValue___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__12; +static lean_object* l_Lean_Elab_Command_mkStructureDecl___lambda__8___closed__1; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__1; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__2; +lean_object* lean_local_ctx_find(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__14; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_replace_expr(lean_object*, lean_object*); +lean_object* l_Lean_LocalDecl_setUserName(lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_ensureNoUnassignedMVars(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_filterMapM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___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_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent_copyFields___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__4___closed__4; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_mkStructureDecl___spec__3(lean_object*, size_t, size_t, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__3; lean_object* lean_st_ref_take(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectLevelParamsInStructure___closed__1; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__10; -lean_object* l_liftExcept___at_Lean_Elab_liftMacroM___spec__1(lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__19; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__12; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__12; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__23; -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__3___boxed(lean_object*, lean_object*, lean_object*, 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_Elab_Command_mkStructureDecl___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*); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___closed__1; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__14; lean_object* l_Lean_Meta_withLetDecl___at_Lean_Elab_Term_elabLetDeclAux___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectLevelParamsInFVars(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Elab_getDeclarationSelectionRef(lean_object*); +static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__9; uint8_t lean_expr_eqv(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__3; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_levelMVarToParam___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_PersistentHashMap_insert___at_Lean_LocalContext_mkLocalDecl___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields_go___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_ResolveName_resolveNamespace(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__8(lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__2; +static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__17; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___closed__2; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__17; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields_go(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__4___closed__2; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___boxed(lean_object**); static lean_object* l_panic___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___spec__1___closed__1; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__20; @@ -391,157 +369,127 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidFieldModifier___lambda__1 lean_object* l_Lean_Core_instantiateValueLevelParams(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Elab_Modifiers_isProtected(lean_object*); lean_object* lean_nat_to_int(lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__12; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__5; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getNestedProjectionArg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__19; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withUsed___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_defaultCtorName___closed__1; -lean_object* l_Lean_MessageData_ofSyntax(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*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___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_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___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___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections(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_Structure_0__Lean_Elab_Command_addProjections(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_mkInductiveType___lambda__3___closed__2; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4___closed__3; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__6(lean_object*, size_t, size_t, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__8; 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_List_forM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__5; static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___closed__1; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__5; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidFieldModifier___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_registerStructure(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__13; -LEAN_EXPORT lean_object* l_Lean_ofExceptKernelException___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___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_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__9; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_go_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_registerTraceClass(lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_StructFieldKind_toCtorIdx(uint8_t); -LEAN_EXPORT lean_object* l_Lean_throwKernelException___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalContext_setBinderInfo(lean_object*, lean_object*, uint8_t); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__4___closed__2; -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___lambda__2(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Elab_Command_getRef(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2___closed__4; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__6___boxed(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__5___closed__6; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___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_setReducibilityStatus___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent_copyFields___spec__2___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields_go___spec__2___closed__7; lean_object* l_Lean_mkCasesOn(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__3___closed__1; 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_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547_(lean_object*, lean_object*); -lean_object* l_Lean_Elab_toAttributeKind___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___closed__4; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__9___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwKernelException___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(lean_object*, lean_object*); 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___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___closed__4; -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__7; -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__19; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___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_Syntax_getKind(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofFormat(lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, 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_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__13; lean_object* l_Lean_Elab_getBetterRef(lean_object*, lean_object*); -lean_object* l_Lean_Elab_expandDeclId___at_Lean_Elab_Term_expandDeclId___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___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_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__1; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___closed__4; lean_object* l_Lean_assignLevelMVar___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent_copyFields___spec__2___lambda__2___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_defaultCtorName___closed__2; -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addCtorFields(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_value(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectLevelParamsInStructure(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___closed__3; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__3; lean_object* l_Lean_Meta_transform___at_Lean_Meta_zetaReduce___spec__1(lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__10; lean_object* l_Lean_Meta_getLevel(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_reduceProjOf_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_forallE___override(lean_object*, lean_object*, lean_object*, uint8_t); lean_object* l_outOfBounds___rarg(lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___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*); -static lean_object* l_Lean_Elab_Command_elabStructure___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor(lean_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_elabParents_go___rarg___lambda__3___boxed(lean_object**); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__8; static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___closed__2; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___spec__1(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields_go___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* l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__1(lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__14; +static lean_object* l_Lean_Elab_Command_instInhabitedStructCtorView___closed__3; +lean_object* l_List_mapTR_loop___at_Lean_Meta_Match_mkMatcher___spec__6(lean_object*, lean_object*); static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4___closed__2; lean_object* lean_st_ref_get(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1___lambda__1___closed__1; -LEAN_EXPORT uint8_t l___private_Lean_Elab_Structure_0__Lean_Elab_Command_validStructType(lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___closed__2; lean_object* l_Lean_Expr_inferImplicit(lean_object*, lean_object*, uint8_t); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkAppM(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__5; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_removeUnused(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_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_Command_StructFieldKind_ofNat(lean_object*); -lean_object* l_List_forM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__6; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkInductiveType___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___closed__1; -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__4; -LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___boxed(lean_object*); -lean_object* l_Lean_Syntax_getOptional_x3f(lean_object*); lean_object* lean_st_mk_ref(lean_object*, lean_object*); -static size_t l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__4; -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__7; +static uint8_t l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__4; lean_object* lean_array_to_list(lean_object*); lean_object* lean_mk_projections(lean_object*, lean_object*, lean_object*, uint8_t); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__21; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabFieldTypeValue___lambda__2___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__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*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__8; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCtor___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_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__17; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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_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___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__6; LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__8___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__3; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__5; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__5; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__6; lean_object* l_Lean_Elab_applyVisibility___at_Lean_Elab_Term_expandDeclId___spec__5(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f(lean_object*, lean_object*); 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_object* l_Lean_Name_append(lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_getFVarLocalDecl_x21(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__4; -static lean_object* l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1___closed__2; -static lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__1; -static lean_object* l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1___closed__1; -static lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__1___closed__2; +static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__7; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_StructFieldKind_noConfusion___rarg(uint8_t, uint8_t, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__10(lean_object*, size_t, size_t, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__2; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___closed__6; -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__5___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__15(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__11; lean_object* l_Lean_Meta_mkId(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_DerivingClassView_applyHandlers(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__2; static lean_object* l_Lean_Elab_Command_checkValidFieldModifier___lambda__3___closed__1; extern lean_object* l_Lean_levelZero; lean_object* l_Lean_Elab_Command_shouldInferResultUniverse(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_expandDeclSig(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__3___boxed(lean_object**); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___lambda__1___boxed(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_mkInductiveType___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_StructFieldKind_noConfusion___rarg___lambda__1___boxed(lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__4; lean_object* l_Lean_Meta_mkInjectiveTheorems(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -549,264 +497,238 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_ge static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__2; lean_object* l_Lean_Meta_whnfD(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_panic___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent_copyFields___spec__1___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); 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*); -lean_object* l_Lean_throwError___at_Lean_Elab_Term_tryPostponeIfHasMVars___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_RBNode_insert___at_Lean_NameMap_insert___spec__1___rarg(lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Elab_Command_getCurrMacroScope(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__7; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_BinderInfo_isInstImplicit(uint8_t); -static lean_object* l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__2; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__1; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addCtorFields___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_panic___at_Lean_Expr_appFn_x21___spec__1(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent_copyFields___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkInductiveType___lambda__3___closed__1; lean_object* l_Lean_Syntax_getSepArgs(lean_object*); lean_object* l_Lean_addMacroScope(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkInductiveType___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidFieldModifier___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_Command_instInhabitedElabStructHeaderResult___closed__3; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields_go___spec__2___closed__4; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__6; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withStructureLocalDecl___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_Command_elabStructureViewPostprocessing(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructureView(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabFieldTypeValue___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_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__5(lean_object*); +static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__8; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields_go___spec__2___closed__2; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectLevelParamsInStructure___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_name_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent_copyFields___spec__2___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___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___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__24; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_getLevelNames___rarg(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__1___closed__2; +static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__5; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkInductiveType___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_Structure_0__Lean_Elab_Command_expandCtor___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__9; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__20; LEAN_EXPORT lean_object* l_Lean_Elab_Command_instReprStructFieldKind; -static lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__7; -LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__2; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUsed___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Term_processDefDeriving___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___lambda__4___boxed(lean_object**); lean_object* l_Lean_Syntax_node2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static size_t l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__5; static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__4; +static lean_object* l_Lean_Elab_Command_structureSyntaxToView___closed__6; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_structureSyntaxToView___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_Structure_0__Lean_Elab_Command_mkTypeFor___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__18; -static lean_object* l_Lean_Elab_Command_elabStructure___closed__8; -static lean_object* l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_instInhabitedElabStructHeaderResult; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields_go___spec__2___closed__10; lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkProjections___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__2; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent_copyFields___spec__2___lambda__2___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__5___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_mkFreshExprMVarImpl(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1___lambda__1___closed__2; -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__2___boxed(lean_object**); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields_go___spec__2___lambda__1___closed__1; -lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__18; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_containsFieldName___boxed(lean_object*, lean_object*); +lean_object* l_Lean_Level_mvarId_x21(lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__16(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__25; +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_object*); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__1; +lean_object* l_Lean_LocalDecl_fvarId(lean_object*); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__11; lean_object* l___private_Lean_ReducibilityAttrs_0__Lean_setReducibilityStatusCore(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__18; +static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__4; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__3; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___closed__4; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent_copyFields___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_withSynthesizeImp___rarg(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_processOveriddenDefaultValues___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_logAt___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__6; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4___closed__5; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__3; lean_object* l_Lean_Elab_Term_withAutoBoundImplicitForbiddenPred___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__1; LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___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_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___closed__2; static lean_object* l_Lean_Elab_Command_StructFieldKind_noConfusion___rarg___closed__1; -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ofExceptKernelException___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___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_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_panic___at_Lean_mkNoConfusionEnum_mkToCtorIdx___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___lambda__2___boxed(lean_object**); -static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__4; static lean_object* l_Lean_Elab_Command_checkValidFieldModifier___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__7___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__3; -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__12; -static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__11; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__12; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields_go___spec__2___closed__6; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructureViewPostprocessing___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_Command_instReprStructFieldInfo; lean_object* l_Lean_Meta_instInhabitedMetaM___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__8; lean_object* l_Lean_addDocString_x27___at_Lean_Elab_Term_expandDeclId___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27___lambda__1___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__13; lean_object* l_Array_append___rarg(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_removeUnused___closed__2; -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___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Elab_Term_applyAttributesAt___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_Environment_contains(lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__4___closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofExpr(lean_object*); lean_object* l_Lean_Option_register___at_Lean_Elab_initFn____x40_Lean_Elab_AutoBound___hyg_6____spec__1(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ofExceptKernelException___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___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_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__5; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___lambda__5___boxed(lean_object**); uint8_t l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27___spec__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__2(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__1; static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__2; -static lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__4; -static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__2; -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__8; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_replaceFieldInfo___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidFieldModifier___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_throwError___at_Lean_Meta_mkSimpCongrTheorem___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_StructFieldInfo_isFromParent___boxed(lean_object*); -static lean_object* l_Lean_Elab_Command_elabStructure___closed__7; +static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___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*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructureViewPostprocessing___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_Structure_0__Lean_Elab_Command_registerStructure(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__15; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__18; LEAN_EXPORT lean_object* l_Array_filterMapM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___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_Structure_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParamFVar(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__9; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311_(lean_object*); lean_object* l_Lean_LocalDecl_userName(lean_object*); lean_object* l_Lean_Meta_getStructureName(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__11(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_Array_extract___rarg(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_node4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f(lean_object*, 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_elabStructHeader___lambda__5___closed__2; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____boxed(lean_object*, lean_object*); lean_object* lean_name_append_index_after(lean_object*, lean_object*); static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___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_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___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_Lean_Elab_Command_instInhabitedStructView___closed__1; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields_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_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_structureSyntaxToView___spec__1___closed__1; uint8_t l_Lean_Elab_Modifiers_isPrivate(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__3; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__4(lean_object*); -static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2___closed__1; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__14; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields(lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__4; -static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2___closed__3; lean_object* l_Lean_Elab_Term_addTermInfo_x27(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_FileMap_leanPosToLspPos(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_levelMVarToParam___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_Command_elabStructure___lambda__2___boxed(lean_object**); -static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed(lean_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_elabFieldTypeValue(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__2; uint8_t l_Lean_Syntax_isToken(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__2; -static lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_structureSyntaxToView___lambda__1___boxed(lean_object**); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__17; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructureView___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__26; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getResultUniverse(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__6; -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__24; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_hasAnyFVar_visit___at_Lean_Expr_containsFVar___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_defaultCtorName; -static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__4; lean_object* l_Lean_getFieldInfo_x3f(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__12; -static lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___spec__2___closed__2; 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_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5_(lean_object*); lean_object* l_Lean_Elab_Term_addLocalVarInfo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_bindingDomain_x21(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__2; lean_object* l_Lean_mkNoConfusion(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___closed__2; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__11; -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___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___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_getOptDerivingClasses(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___closed__2; +LEAN_EXPORT lean_object* l_List_forM___at_Lean_Elab_Command_mkStructureDecl___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_Structure_0__Lean_Elab_Command_mkAuxConstructions___closed__4; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_elabStructure___closed__1; LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__8___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_instInhabitedStructParentInfo___closed__1; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_Command_StructFieldInfo_isSubobject(lean_object*); extern lean_object* l_Lean_NameSet_empty; +static lean_object* l_Lean_Elab_Command_structureSyntaxToView___closed__7; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructureViewPostprocessing___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__6; +static lean_object* l_Lean_Elab_Command_structureSyntaxToView___closed__9; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent_copyFields___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___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*); lean_object* l_Lean_Expr_app___override(lean_object*, lean_object*); lean_object* lean_string_length(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27___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_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__1; lean_object* l_Lean_Level_getLevelOffset(lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_mkStructureDecl___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl(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_expandFields___closed__4; lean_object* l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabStructureViewPostprocessing___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_getForallBody(lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); lean_object* l_Lean_Meta_mkFreshLevelMVarsFor(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__3___boxed(lean_object**); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__8; static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__1; lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_3025_(lean_object*, lean_object*); lean_object* l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_getFVarLocalDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1(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__14; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_processOveriddenDefaultValues___spec__1(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkToParentName___closed__1; -lean_object* l_Lean_Name_beq___boxed(lean_object*, lean_object*); +lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6(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_Structure_0__Lean_Elab_Command_elabFieldTypeValue___lambda__1___boxed(lean_object*, lean_object*); lean_object* lean_environment_main_module(lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__21; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__12; lean_object* l_Lean_instantiateMVars___at___private_Lean_Meta_Basic_0__Lean_Meta_isClassApp_x3f___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_accLevelAtCtor___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__11(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__5; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__1; +lean_object* l_Lean_MessageData_ofLevel(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUsed___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getNestedProjectionArg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_Command_instInhabitedStructFieldKind; lean_object* l_Lean_Meta_getLocalInstances(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___closed__3; -static lean_object* l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4___closed__2; lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_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_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__2; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__5___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getNestedProjectionArg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_removeUnused___closed__4; lean_object* l_Lean_indentExpr(lean_object*); @@ -814,32 +736,45 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_le LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reduceProjs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__2; uint8_t l_Lean_BinderInfo_isExplicit(uint8_t); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__9; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withStructureLocalDecl___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___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_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*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__4; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields_go___spec__2___closed__8; LEAN_EXPORT uint8_t l___private_Lean_Elab_Structure_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27___lambda__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990_(lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabStructure___spec__3(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__2; lean_object* l_Lean_Syntax_node1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_instInhabitedStructFieldInfo___closed__2; +static lean_object* l_Lean_Elab_Command_structureSyntaxToView___closed__8; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___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 size_t l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__4; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_instInhabitedStructCtorView; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__1; lean_object* l_Lean_Elab_Command_accLevel_go(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkHasTypeButIsExpectedMsg(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*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__2; uint8_t l_Lean_NameSet_contains(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__1(lean_object*, lean_object*); +lean_object* l_Lean_Elab_Term_expandDeclId(lean_object*, 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_setSourceInstImplicit___closed__2; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__7; -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__1___boxed(lean_object**); +lean_object* l_Lean_Linter_logLintIf___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__25(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_copyDefaultValue_x3f_failed___closed__4; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___lambda__7(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go(lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__6(lean_object*, size_t, size_t, lean_object*); +static lean_object* l_Lean_Elab_Command_mkStructureDecl___lambda__5___closed__2; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__11; +lean_object* l_Lean_Meta_forallBoundedTelescope___at_Lean_Elab_Term_addAutoBoundImplicits_x27___spec__2___rarg(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_go_x3f___closed__2; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___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*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___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*); +uint8_t l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__2; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__14; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___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*); +static lean_object* l_Lean_Elab_Command_elabStructure___lambda__2___closed__2; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_type(lean_object*); lean_object* l_Repr_addAppParen(lean_object*, lean_object*); @@ -849,251 +784,468 @@ static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFie LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__5___rarg(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_object* lean_panic_fn(lean_object*, lean_object*); -static lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__2; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__5; static lean_object* l_Lean_Elab_Command_instInhabitedStructFieldInfo___closed__1; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_removeUnused___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_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__13; -static lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__6; -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabStructure___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_ResolveName_resolveGlobalName(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_mkStructureDecl___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*); +static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__12; +LEAN_EXPORT lean_object* l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__16; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__5___boxed(lean_object**); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__6; lean_object* l_Lean_Expr_getAppFn(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields(lean_object*, lean_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___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__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_Structure_0__Lean_Elab_Command_getFieldType___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__10; -LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_addInstance(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Elab_Command_liftCoreM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__3___closed__1; -static lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___closed__2; +uint8_t l_Lean_Expr_isProp(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___lambda__6___boxed(lean_object**); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___closed__2; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_structureSyntaxToView___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*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___spec__2(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_mkStructureDecl___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_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__3; +static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__15; +static lean_object* l_Lean_Elab_Command_instInhabitedStructCtorView___closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents(lean_object*); lean_object* l_Lean_Elab_Term_withoutAutoBoundImplicit___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_isPrivateName(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_StructFieldKind_noConfusion(lean_object*); -static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__4; -static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__3; +static lean_object* l_Lean_Elab_Command_mkStructureDecl___lambda__3___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_instInhabitedStructParentInfo; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkInductiveType___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_Command_structureSyntaxToView___closed__5; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__5; -LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__8; lean_object* l_Lean_Elab_expandOptDeclSig(lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__7; extern lean_object* l_Lean_Linter_linter_deprecated; lean_object* l_Lean_Name_getString_x21(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkToParentName_go(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); -static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__4___closed__3; lean_object* l_Array_ofSubarray___rarg(lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent_copyFields___closed__1; uint8_t l_Lean_LocalDecl_binderInfo(lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___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___private_Lean_Elab_Structure_0__Lean_Elab_Command_levelMVarToParam(lean_object*, lean_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___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_protectedExt; -extern lean_object* l_Lean_instInhabitedDeclarationRanges; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3; lean_object* lean_erase_macro_scopes(lean_object*); +static lean_object* l_Lean_Elab_Command_structureSyntaxToView___closed__4; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__9; -static lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__2___closed__2; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_mkStructureDecl___spec__6(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_Structure_0__Lean_Elab_Command_copyNewFieldsFrom(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___lambda__1___boxed(lean_object*); lean_object* l_List_reverse___rarg(lean_object*); +lean_object* l_Lean_Elab_Term_withAuxDecl___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkAuxDefinition(lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_mkStructureDecl___lambda__5___closed__1; lean_object* lean_array_mk(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getResultUniverse___closed__1; -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___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_Command_StructFieldKind_ofNat___boxed(lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__16; -LEAN_EXPORT lean_object* l_Lean_Linter_logLintIf___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___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_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_removeUnused(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__17; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__9; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__3; +lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__12(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___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkTypeFor(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_toVisibility(lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); +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_Command_instInhabitedStructView; static lean_object* l_Lean_Elab_Command_checkValidFieldModifier___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__2; +static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__18; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__19; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__8; uint8_t l_Lean_Level_isMVar(lean_object*); -static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__1; -static lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__6; -static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__11___closed__1; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__27; lean_object* l_Lean_Elab_Term_withLevelNames___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___closed__1; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__5; static lean_object* l_Lean_Elab_Command_checkValidFieldModifier___lambda__2___closed__2; lean_object* lean_array_uget(lean_object*, size_t); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__1; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_mkStructureDecl___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___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*); size_t lean_array_size(lean_object*); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__7; +static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__8; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withUsed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___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_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__2(lean_object*); -static lean_object* l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__3; -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__3; -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__11; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_structureSyntaxToView___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +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_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_structureSyntaxToView___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___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkToParentName(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_mkStructureDecl___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___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__5___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__7(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__25; -static lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__1___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__19(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__5___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getNestedProjectionArg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__1; lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__7; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___closed__5; -static lean_object* l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__4; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields_go___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_elabStructure___closed__3; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__5___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__1(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_structureSyntaxToView___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_string_append(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_StructFieldKind_noConfusion___rarg___lambda__1(lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___closed__1; lean_object* l_Lean_mkAtomFrom(lean_object*, lean_object*, uint8_t); -lean_object* l_Lean_getAttributeImpl(lean_object*, lean_object*); +lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___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_Structure_0__Lean_Elab_Command_expandFields___closed__6; +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instReprStructFieldKind___closed__1; +LEAN_EXPORT lean_object* l_Lean_ofExceptKernelException___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___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_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__18; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__4___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__4; -static lean_object* l_Lean_Elab_Command_elabStructure___closed__6; +static lean_object* l_Lean_Elab_Command_structureSyntaxToView___closed__3; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_mkStructureDecl___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_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields_go___spec__2___closed__1; -static lean_object* l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__5; -static lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__3___closed__2; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkTypeFor___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_Command_checkValidCtorModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__22(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__3; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__7; lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20(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_addDefaults___spec__2___closed__3; +static lean_object* l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__3; uint8_t lean_nat_dec_le(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__1; -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -extern lean_object* l_Lean_Elab_unsupportedSyntaxExceptionId; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_structureSyntaxToView(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_panic___at_Lean_ResolveName_resolveNamespaceUsingScope_x3f___spec__1(lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___closed__2; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__26; lean_object* l_Lean_RBNode_find___at_Lean_NameMap_find_x3f___spec__1___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2___closed__2; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__6; uint8_t l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_404_(uint8_t, uint8_t); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__9; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUsed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__2; lean_object* l_Lean_Meta_mkLambdaFVars(lean_object*, lean_object*, uint8_t, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkProjection(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_expandFields___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent_copyFields___spec__2___closed__4; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUsed___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_addAndCompile(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_elabStructure___closed__5; lean_object* lean_nat_add(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__5; -LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__23; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__2; -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__7(lean_object*, size_t, size_t, lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__5; LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent_copyFields___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__24; -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_List_mapTR_loop___at_Lean_compileDecl___spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__15; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateFieldInfoVal(lean_object*, lean_object*, lean_object*); -uint8_t l_Lean_Exception_isRuntime(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___lambda__1(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__4___closed__1; -LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkConstWithLevelParams___at_Lean_Elab_Term_expandDeclId___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__5; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___spec__2___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields___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_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__3; uint8_t l_Lean_Expr_isFVar(lean_object*); uint8_t l_Lean_Expr_isForall(lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__10; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___lambda__4___boxed(lean_object**); -lean_object* l_Lean_expandMacros(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___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_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_replaceFieldInfo(lean_object*, lean_object*); lean_object* l_Lean_getStructureFieldsFlattened(lean_object*, lean_object*, uint8_t); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___lambda__5(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__10; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___closed__1; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_mkStructureDecl___spec__4(lean_object*, size_t, size_t, lean_object*); lean_object* l_Lean_KernelException_toMessageData(lean_object*, lean_object*); uint8_t lean_is_class(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__6; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields_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_Lean_throwKernelException___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_String_toSubstring_x27(lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__2; -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___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_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___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_Elab_Structure_0__Lean_Elab_Command_withFields_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*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___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_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_mkCoercionToCopiedParent___lambda__1___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__24; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent_copyFields___spec__2___closed__3; lean_object* l_Lean_logWarning___at_Lean_Elab_Term_mkConst___spec__4(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___private_Lean_Elab_Structure_0__Lean_Elab_Command_removeUnused___closed__3; -static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___closed__3; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___lambda__1___boxed(lean_object**); lean_object* l_Lean_MessageData_ofName(lean_object*); -static uint8_t l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__2; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__2; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__5; lean_object* lean_expr_instantiate1(lean_object*, lean_object*); +lean_object* l___private_Init_Data_Repr_0__Nat_reprFast(lean_object*); uint8_t l_Lean_Elab_Modifiers_isPartial(lean_object*); +static lean_object* l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__7; lean_object* l_mkRecOn(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__7; -static lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___closed__1; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__16; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); 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_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__9(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_structureSyntaxToView___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_collectFVars(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent_copyFields___spec__2___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reduceProjs___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__1___boxed(lean_object**); -static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__7; -LEAN_EXPORT lean_object* l_Lean_Linter_logLintIf___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__18(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_isProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addDecl(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_elabType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__28; LEAN_EXPORT lean_object* l_Lean_setReducibilityStatus___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__1(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_ReaderT_pure___at_Lean_Elab_liftMacroM___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___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___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent_copyFields___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___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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_Command_elabStructure___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__1; +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__12; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__10; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___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_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___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__4___closed__1; uint8_t l_Lean_Expr_hasExprMVar(lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Array_isEmpty___rarg(lean_object*); -LEAN_EXPORT uint8_t l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___lambda__1(lean_object*, lean_object*, lean_object*); lean_object* l_Array_get_x3f___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Level_getOffsetAux(lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_withDeclName___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("structureDiamondWarning", 23, 23); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("", 0, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("enable/disable warning messages for structure diamonds", 54, 54); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__5() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = 0; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__3; +x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__4; +x_4 = lean_box(x_1); +x_5 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_5, 0, x_4); +lean_ctor_set(x_5, 1, x_2); +lean_ctor_set(x_5, 2, x_3); +return x_5; +} +} +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__7() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Elab", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__8() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Command", 7, 7); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__9() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__6; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__7; +x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__8; +x_4 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__1; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__2; +x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__5; +x_4 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__9; +x_5 = l_Lean_Option_register___at_Lean_Elab_initFn____x40_Lean_Elab_AutoBound___hyg_6____spec__1(x_2, x_3, x_4, x_1); +return x_5; +} +} +static lean_object* _init_l_Lean_Elab_Command_instInhabitedStructCtorView___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_Elab_Command_instInhabitedStructCtorView___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; uint8_t x_5; lean_object* x_6; lean_object* x_7; +x_1 = lean_box(0); +x_2 = lean_box(0); +x_3 = 0; +x_4 = 0; +x_5 = 0; +x_6 = l_Lean_Elab_Command_instInhabitedStructCtorView___closed__1; +x_7 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_7, 0, x_2); +lean_ctor_set(x_7, 1, x_1); +lean_ctor_set(x_7, 2, x_6); +lean_ctor_set_uint8(x_7, sizeof(void*)*3, x_3); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 1, x_4); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 2, x_5); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 3, x_4); +return x_7; +} +} +static lean_object* _init_l_Lean_Elab_Command_instInhabitedStructCtorView___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Command_instInhabitedStructCtorView___closed__2; +x_3 = lean_box(0); +x_4 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +lean_ctor_set(x_4, 3, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_Elab_Command_instInhabitedStructCtorView() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Elab_Command_instInhabitedStructCtorView___closed__3; +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Command_instInhabitedStructView___closed__1() { +_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; lean_object* x_7; lean_object* x_8; +x_1 = lean_box(0); +x_2 = lean_box(0); +x_3 = l_Lean_Elab_Command_instInhabitedStructCtorView___closed__2; +x_4 = 0; +x_5 = lean_box(0); +x_6 = l_Lean_Elab_Command_instInhabitedStructCtorView___closed__1; +x_7 = l_Lean_Elab_Command_instInhabitedStructCtorView___closed__3; +x_8 = lean_alloc_ctor(0, 12, 1); +lean_ctor_set(x_8, 0, x_2); +lean_ctor_set(x_8, 1, x_2); +lean_ctor_set(x_8, 2, x_3); +lean_ctor_set(x_8, 3, x_5); +lean_ctor_set(x_8, 4, x_5); +lean_ctor_set(x_8, 5, x_1); +lean_ctor_set(x_8, 6, x_2); +lean_ctor_set(x_8, 7, x_2); +lean_ctor_set(x_8, 8, x_6); +lean_ctor_set(x_8, 9, x_7); +lean_ctor_set(x_8, 10, x_6); +lean_ctor_set(x_8, 11, x_6); +lean_ctor_set_uint8(x_8, sizeof(void*)*12, x_4); +return x_8; +} +} +static lean_object* _init_l_Lean_Elab_Command_instInhabitedStructView() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Elab_Command_instInhabitedStructView___closed__1; +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Command_instInhabitedStructParentInfo___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(0u); +x_2 = l_Lean_Expr_bvar___override(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Command_instInhabitedStructParentInfo___closed__2() { +_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 = lean_box(0); +x_2 = lean_box(0); +x_3 = lean_box(0); +x_4 = 0; +x_5 = l_Lean_Elab_Command_instInhabitedStructParentInfo___closed__1; +x_6 = lean_alloc_ctor(0, 4, 1); +lean_ctor_set(x_6, 0, x_2); +lean_ctor_set(x_6, 1, x_1); +lean_ctor_set(x_6, 2, x_3); +lean_ctor_set(x_6, 3, x_5); +lean_ctor_set_uint8(x_6, sizeof(void*)*4, x_4); +return x_6; +} +} +static lean_object* _init_l_Lean_Elab_Command_instInhabitedStructParentInfo() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Elab_Command_instInhabitedStructParentInfo___closed__2; +return x_1; +} +} LEAN_EXPORT lean_object* l_Lean_Elab_Command_StructFieldKind_toCtorIdx(uint8_t x_1) { _start: { @@ -1273,7 +1425,7 @@ x_6 = lean_box(x_5); return x_6; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__1() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__1() { _start: { lean_object* x_1; @@ -1281,17 +1433,17 @@ x_1 = lean_mk_string_unchecked("Lean.Elab.Command.StructFieldKind.newField", 42, return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__2() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__1; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__1; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__3() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__3() { _start: { lean_object* x_1; lean_object* x_2; @@ -1300,23 +1452,23 @@ x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__4() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__3; -x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__2; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__3; +x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__2; x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__5() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__5() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__4; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__4; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -1324,7 +1476,7 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__6() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__6() { _start: { lean_object* x_1; lean_object* x_2; @@ -1333,23 +1485,23 @@ x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__7() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__6; -x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__2; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__6; +x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__2; x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__8() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__8() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__7; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__7; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -1357,7 +1509,7 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__9() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__9() { _start: { lean_object* x_1; @@ -1365,33 +1517,33 @@ x_1 = lean_mk_string_unchecked("Lean.Elab.Command.StructFieldKind.copiedField", return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__10() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__10() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__9; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__9; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__11() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__3; -x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__10; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__3; +x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__10; x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__12() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__12() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__11; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__11; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -1399,23 +1551,23 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__13() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__6; -x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__10; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__6; +x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__10; x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__14() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__14() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__13; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__13; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -1423,7 +1575,7 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__15() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__15() { _start: { lean_object* x_1; @@ -1431,33 +1583,33 @@ x_1 = lean_mk_string_unchecked("Lean.Elab.Command.StructFieldKind.fromParent", 4 return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__16() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__16() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__15; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____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_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__17() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__17() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__3; -x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__16; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__3; +x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__16; x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__18() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__18() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__17; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__17; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -1465,23 +1617,23 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__19() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__19() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__6; -x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__16; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__6; +x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__16; x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__20() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__20() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__19; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__19; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -1489,7 +1641,7 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__21() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__21() { _start: { lean_object* x_1; @@ -1497,33 +1649,33 @@ x_1 = lean_mk_string_unchecked("Lean.Elab.Command.StructFieldKind.subobject", 43 return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__22() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__22() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__21; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__21; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__23() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__23() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__3; -x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__22; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__3; +x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__22; x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__24() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__24() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__23; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__23; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -1531,23 +1683,23 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__25() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__25() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__6; -x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__22; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__6; +x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__22; x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__26() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__26() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__25; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__25; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -1555,7 +1707,7 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339_(uint8_t x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481_(uint8_t x_1, lean_object* x_2) { _start: { switch (x_1) { @@ -1567,14 +1719,14 @@ x_4 = lean_nat_dec_le(x_3, x_2); if (x_4 == 0) { lean_object* x_5; lean_object* x_6; -x_5 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__5; +x_5 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__5; x_6 = l_Repr_addAppParen(x_5, x_2); return x_6; } else { lean_object* x_7; lean_object* x_8; -x_7 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__8; +x_7 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__8; x_8 = l_Repr_addAppParen(x_7, x_2); return x_8; } @@ -1587,14 +1739,14 @@ x_10 = lean_nat_dec_le(x_9, x_2); if (x_10 == 0) { lean_object* x_11; lean_object* x_12; -x_11 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__12; +x_11 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__12; x_12 = l_Repr_addAppParen(x_11, x_2); return x_12; } else { lean_object* x_13; lean_object* x_14; -x_13 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__14; +x_13 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__14; x_14 = l_Repr_addAppParen(x_13, x_2); return x_14; } @@ -1607,14 +1759,14 @@ x_16 = lean_nat_dec_le(x_15, x_2); if (x_16 == 0) { lean_object* x_17; lean_object* x_18; -x_17 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__18; +x_17 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__18; x_18 = l_Repr_addAppParen(x_17, x_2); return x_18; } else { lean_object* x_19; lean_object* x_20; -x_19 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__20; +x_19 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__20; x_20 = l_Repr_addAppParen(x_19, x_2); return x_20; } @@ -1627,14 +1779,14 @@ x_22 = lean_nat_dec_le(x_21, x_2); if (x_22 == 0) { lean_object* x_23; lean_object* x_24; -x_23 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__24; +x_23 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__24; x_24 = l_Repr_addAppParen(x_23, x_2); return x_24; } else { lean_object* x_25; lean_object* x_26; -x_25 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__26; +x_25 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__26; x_26 = l_Repr_addAppParen(x_25, x_2); return x_26; } @@ -1642,13 +1794,13 @@ return x_26; } } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; x_3 = lean_unbox(x_1); lean_dec(x_1); -x_4 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339_(x_3, x_2); +x_4 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481_(x_3, x_2); lean_dec(x_2); return x_4; } @@ -1657,7 +1809,7 @@ static lean_object* _init_l_Lean_Elab_Command_instReprStructFieldKind___closed__ _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____boxed), 2, 0); return x_1; } } @@ -1672,68 +1824,61 @@ return x_1; static lean_object* _init_l_Lean_Elab_Command_instInhabitedStructFieldInfo___closed__1() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(0u); -x_2 = l_Lean_Expr_bvar___override(x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Elab_Command_instInhabitedStructFieldInfo___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; uint8_t x_5; lean_object* x_6; x_1 = lean_box(0); x_2 = lean_box(0); -x_3 = l_Lean_Elab_Command_instInhabitedStructFieldInfo___closed__1; -x_4 = 0; -x_5 = lean_alloc_ctor(0, 4, 1); -lean_ctor_set(x_5, 0, x_2); -lean_ctor_set(x_5, 1, x_2); -lean_ctor_set(x_5, 2, x_3); -lean_ctor_set(x_5, 3, x_1); -lean_ctor_set_uint8(x_5, sizeof(void*)*4, x_4); -return x_5; +x_3 = lean_box(0); +x_4 = l_Lean_Elab_Command_instInhabitedStructParentInfo___closed__1; +x_5 = 0; +x_6 = lean_alloc_ctor(0, 5, 1); +lean_ctor_set(x_6, 0, x_2); +lean_ctor_set(x_6, 1, x_3); +lean_ctor_set(x_6, 2, x_3); +lean_ctor_set(x_6, 3, x_4); +lean_ctor_set(x_6, 4, x_1); +lean_ctor_set_uint8(x_6, sizeof(void*)*5, x_5); +return x_6; } } static lean_object* _init_l_Lean_Elab_Command_instInhabitedStructFieldInfo() { _start: { lean_object* x_1; -x_1 = l_Lean_Elab_Command_instInhabitedStructFieldInfo___closed__2; +x_1 = l_Lean_Elab_Command_instInhabitedStructFieldInfo___closed__1; return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__1() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("name", 4, 4); +x_1 = lean_mk_string_unchecked("ref", 3, 3); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__2() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__1; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__1; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__3() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__2; +x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__2; x_3 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__4() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__4() { _start: { lean_object* x_1; @@ -1741,38 +1886,38 @@ x_1 = lean_mk_string_unchecked(" := ", 4, 4); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__5() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__5() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__4; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__4; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__6() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__3; -x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__5; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__3; +x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__5; x_3 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__7() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__7() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(8u); +x_1 = lean_unsigned_to_nat(7u); x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__8() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__8() { _start: { lean_object* x_1; @@ -1780,17 +1925,44 @@ x_1 = lean_mk_string_unchecked(",", 1, 1); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__9() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__9() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__8; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__10() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("name", 4, 4); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__11() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__8; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__10; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__10() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__12() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(8u); +x_2 = lean_nat_to_int(x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__13() { _start: { lean_object* x_1; @@ -1798,17 +1970,17 @@ x_1 = lean_mk_string_unchecked("declName", 8, 8); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__11() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__14() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__10; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____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_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__12() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__15() { _start: { lean_object* x_1; lean_object* x_2; @@ -1817,7 +1989,7 @@ x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__13() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__16() { _start: { lean_object* x_1; @@ -1825,17 +1997,17 @@ x_1 = lean_mk_string_unchecked("fvar", 4, 4); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__14() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__17() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__13; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__16; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__15() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__18() { _start: { lean_object* x_1; @@ -1843,17 +2015,17 @@ x_1 = lean_mk_string_unchecked("kind", 4, 4); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__16() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__19() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__15; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__18; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__17() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__20() { _start: { lean_object* x_1; @@ -1861,17 +2033,17 @@ x_1 = lean_mk_string_unchecked("value\?", 6, 6); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__18() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__21() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__17; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__20; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__19() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__22() { _start: { lean_object* x_1; lean_object* x_2; @@ -1880,7 +2052,7 @@ x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__20() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__23() { _start: { lean_object* x_1; @@ -1888,35 +2060,35 @@ x_1 = lean_mk_string_unchecked("{ ", 2, 2); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__21() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__24() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__20; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__23; x_2 = lean_string_length(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__22() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__25() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__21; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__24; x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__23() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__26() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__20; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____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_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__24() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__27() { _start: { lean_object* x_1; @@ -1924,25 +2096,25 @@ x_1 = lean_mk_string_unchecked(" }", 2, 2); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__25() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__28() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__24; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__27; 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_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547_(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698_(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; uint8_t x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; x_3 = lean_ctor_get(x_1, 0); lean_inc(x_3); x_4 = lean_unsigned_to_nat(0u); -x_5 = l_Lean_Name_reprPrec(x_3, x_4); -x_6 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__7; +x_5 = l___private_Init_Meta_0__Lean_Syntax_reprSyntax____x40_Init_Meta___hyg_2168_(x_3, x_4); +x_6 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__7; x_7 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_7, 0, x_6); lean_ctor_set(x_7, 1, x_5); @@ -1950,11 +2122,11 @@ x_8 = 0; x_9 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_9, 0, x_7); lean_ctor_set_uint8(x_9, sizeof(void*)*1, x_8); -x_10 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__6; +x_10 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__6; x_11 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_11, 0, x_10); lean_ctor_set(x_11, 1, x_9); -x_12 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__9; +x_12 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__9; x_13 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_13, 0, x_11); lean_ctor_set(x_13, 1, x_12); @@ -1962,18 +2134,18 @@ x_14 = lean_box(1); x_15 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_15, 0, x_13); lean_ctor_set(x_15, 1, x_14); -x_16 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__11; +x_16 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__11; x_17 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_17, 0, x_15); lean_ctor_set(x_17, 1, x_16); -x_18 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__5; +x_18 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__5; x_19 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_19, 0, x_17); lean_ctor_set(x_19, 1, x_18); x_20 = lean_ctor_get(x_1, 1); lean_inc(x_20); x_21 = l_Lean_Name_reprPrec(x_20, x_4); -x_22 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__12; +x_22 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__12; x_23 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_23, 0, x_22); lean_ctor_set(x_23, 1, x_21); @@ -1989,7 +2161,7 @@ lean_ctor_set(x_26, 1, x_12); x_27 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_27, 0, x_26); lean_ctor_set(x_27, 1, x_14); -x_28 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__14; +x_28 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__14; x_29 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_29, 0, x_27); lean_ctor_set(x_29, 1, x_28); @@ -1998,90 +2170,116 @@ lean_ctor_set(x_30, 0, x_29); lean_ctor_set(x_30, 1, x_18); x_31 = lean_ctor_get(x_1, 2); lean_inc(x_31); -x_32 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_3025_(x_31, x_4); -x_33 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_33, 0, x_6); -lean_ctor_set(x_33, 1, x_32); -x_34 = lean_alloc_ctor(6, 1, 1); +x_32 = l_Lean_Name_reprPrec(x_31, x_4); +x_33 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__15; +x_34 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_34, 0, x_33); -lean_ctor_set_uint8(x_34, sizeof(void*)*1, x_8); -x_35 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_35, 0, x_30); -lean_ctor_set(x_35, 1, x_34); +lean_ctor_set(x_34, 1, x_32); +x_35 = lean_alloc_ctor(6, 1, 1); +lean_ctor_set(x_35, 0, x_34); +lean_ctor_set_uint8(x_35, sizeof(void*)*1, x_8); x_36 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_36, 0, x_35); -lean_ctor_set(x_36, 1, x_12); +lean_ctor_set(x_36, 0, x_30); +lean_ctor_set(x_36, 1, x_35); x_37 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_37, 0, x_36); -lean_ctor_set(x_37, 1, x_14); -x_38 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__16; -x_39 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_39, 0, x_37); -lean_ctor_set(x_39, 1, x_38); +lean_ctor_set(x_37, 1, x_12); +x_38 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_38, 0, x_37); +lean_ctor_set(x_38, 1, x_14); +x_39 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__17; x_40 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_40, 0, x_39); -lean_ctor_set(x_40, 1, x_18); -x_41 = lean_ctor_get_uint8(x_1, sizeof(void*)*4); -x_42 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339_(x_41, x_4); -x_43 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_43, 0, x_6); -lean_ctor_set(x_43, 1, x_42); -x_44 = lean_alloc_ctor(6, 1, 1); -lean_ctor_set(x_44, 0, x_43); -lean_ctor_set_uint8(x_44, sizeof(void*)*1, x_8); -x_45 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_45, 0, x_40); -lean_ctor_set(x_45, 1, x_44); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +x_41 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_41, 0, x_40); +lean_ctor_set(x_41, 1, x_18); +x_42 = lean_ctor_get(x_1, 3); +lean_inc(x_42); +x_43 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_3025_(x_42, x_4); +x_44 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_44, 0, x_22); +lean_ctor_set(x_44, 1, x_43); +x_45 = lean_alloc_ctor(6, 1, 1); +lean_ctor_set(x_45, 0, x_44); +lean_ctor_set_uint8(x_45, sizeof(void*)*1, x_8); x_46 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_46, 0, x_45); -lean_ctor_set(x_46, 1, x_12); +lean_ctor_set(x_46, 0, x_41); +lean_ctor_set(x_46, 1, x_45); x_47 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_47, 0, x_46); -lean_ctor_set(x_47, 1, x_14); -x_48 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__18; -x_49 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_49, 0, x_47); -lean_ctor_set(x_49, 1, x_48); +lean_ctor_set(x_47, 1, x_12); +x_48 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_48, 0, x_47); +lean_ctor_set(x_48, 1, x_14); +x_49 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__19; x_50 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_50, 0, x_49); -lean_ctor_set(x_50, 1, x_18); -x_51 = lean_ctor_get(x_1, 3); -lean_inc(x_51); -lean_dec(x_1); -x_52 = l_Option_repr___at___private_Lean_Meta_Transform_0__Lean_reprTransformStep____x40_Lean_Meta_Transform___hyg_45____spec__1(x_51, x_4); -x_53 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__19; +lean_ctor_set(x_50, 0, x_48); +lean_ctor_set(x_50, 1, x_49); +x_51 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_51, 0, x_50); +lean_ctor_set(x_51, 1, x_18); +x_52 = lean_ctor_get_uint8(x_1, sizeof(void*)*5); +x_53 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481_(x_52, x_4); x_54 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_54, 0, x_53); -lean_ctor_set(x_54, 1, x_52); +lean_ctor_set(x_54, 0, x_22); +lean_ctor_set(x_54, 1, x_53); x_55 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_55, 0, x_54); lean_ctor_set_uint8(x_55, sizeof(void*)*1, x_8); x_56 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_56, 0, x_50); +lean_ctor_set(x_56, 0, x_51); lean_ctor_set(x_56, 1, x_55); -x_57 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__23; +x_57 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_57, 0, x_56); +lean_ctor_set(x_57, 1, x_12); x_58 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_58, 0, x_57); -lean_ctor_set(x_58, 1, x_56); -x_59 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__25; +lean_ctor_set(x_58, 1, x_14); +x_59 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__21; x_60 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_60, 0, x_58); lean_ctor_set(x_60, 1, x_59); -x_61 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__22; -x_62 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_62, 0, x_61); -lean_ctor_set(x_62, 1, x_60); -x_63 = lean_alloc_ctor(6, 1, 1); -lean_ctor_set(x_63, 0, x_62); -lean_ctor_set_uint8(x_63, sizeof(void*)*1, x_8); -return x_63; +x_61 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_61, 0, x_60); +lean_ctor_set(x_61, 1, x_18); +x_62 = lean_ctor_get(x_1, 4); +lean_inc(x_62); +lean_dec(x_1); +x_63 = l_Option_repr___at___private_Lean_Meta_Transform_0__Lean_reprTransformStep____x40_Lean_Meta_Transform___hyg_45____spec__1(x_62, x_4); +x_64 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__22; +x_65 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_65, 0, x_64); +lean_ctor_set(x_65, 1, x_63); +x_66 = lean_alloc_ctor(6, 1, 1); +lean_ctor_set(x_66, 0, x_65); +lean_ctor_set_uint8(x_66, sizeof(void*)*1, x_8); +x_67 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_67, 0, x_61); +lean_ctor_set(x_67, 1, x_66); +x_68 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__26; +x_69 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_69, 0, x_68); +lean_ctor_set(x_69, 1, x_67); +x_70 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__28; +x_71 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_71, 0, x_69); +lean_ctor_set(x_71, 1, x_70); +x_72 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__25; +x_73 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_73, 0, x_72); +lean_ctor_set(x_73, 1, x_71); +x_74 = lean_alloc_ctor(6, 1, 1); +lean_ctor_set(x_74, 0, x_73); +lean_ctor_set_uint8(x_74, sizeof(void*)*1, x_8); +return x_74; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547_(x_1, x_2); +x_3 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698_(x_1, x_2); lean_dec(x_2); return x_3; } @@ -2090,7 +2288,7 @@ static lean_object* _init_l_Lean_Elab_Command_instReprStructFieldInfo___closed__ _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____boxed), 2, 0); return x_1; } } @@ -2102,22 +2300,117 @@ x_1 = l_Lean_Elab_Command_instReprStructFieldInfo___closed__1; return x_1; } } -LEAN_EXPORT uint8_t l_Lean_Elab_Command_StructFieldInfo_isFromParent(lean_object* x_1) { +static lean_object* _init_l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__1() { _start: { -uint8_t x_2; lean_object* x_3; -x_2 = lean_ctor_get_uint8(x_1, sizeof(void*)*4); -x_3 = lean_box(x_2); -if (lean_obj_tag(x_3) == 2) -{ -uint8_t x_4; -x_4 = 1; -return x_4; +lean_object* x_1; +x_1 = l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_box(0), lean_box(0)); +return x_1; } -else +} +static lean_object* _init_l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__2() { +_start: { -uint8_t x_5; -lean_dec(x_3); +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__1; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_instInhabitedStructCtorView___closed__1; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static size_t _init_l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__4() { +_start: +{ +lean_object* x_1; size_t x_2; +x_1 = lean_unsigned_to_nat(0u); +x_2 = lean_usize_of_nat(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; size_t x_4; lean_object* x_5; +x_1 = l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__3; +x_2 = l_Lean_Elab_Command_instInhabitedStructCtorView___closed__1; +x_3 = lean_unsigned_to_nat(0u); +x_4 = l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__4; +x_5 = lean_alloc_ctor(0, 4, sizeof(size_t)*1); +lean_ctor_set(x_5, 0, x_1); +lean_ctor_set(x_5, 1, x_2); +lean_ctor_set(x_5, 2, x_3); +lean_ctor_set(x_5, 3, x_3); +lean_ctor_set_usize(x_5, 4, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__2; +x_2 = l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__5; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Command_instInhabitedStructView___closed__1; +x_3 = l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__6; +x_4 = l_Lean_Elab_Command_instInhabitedStructCtorView___closed__1; +x_5 = l_Lean_Elab_Command_instInhabitedStructParentInfo___closed__1; +x_6 = lean_alloc_ctor(0, 8, 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_1); +lean_ctor_set(x_6, 4, x_4); +lean_ctor_set(x_6, 5, x_5); +lean_ctor_set(x_6, 6, x_4); +lean_ctor_set(x_6, 7, x_4); +return x_6; +} +} +static lean_object* _init_l_Lean_Elab_Command_instInhabitedElabStructHeaderResult() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__7; +return x_1; +} +} +LEAN_EXPORT uint8_t l_Lean_Elab_Command_StructFieldInfo_isFromParent(lean_object* x_1) { +_start: +{ +uint8_t x_2; lean_object* x_3; +x_2 = lean_ctor_get_uint8(x_1, sizeof(void*)*5); +x_3 = lean_box(x_2); +if (lean_obj_tag(x_3) == 2) +{ +uint8_t x_4; +x_4 = 1; +return x_4; +} +else +{ +uint8_t x_5; +lean_dec(x_3); x_5 = 0; return x_5; } @@ -2137,7 +2430,7 @@ LEAN_EXPORT uint8_t l_Lean_Elab_Command_StructFieldInfo_isSubobject(lean_object* _start: { uint8_t x_2; lean_object* x_3; -x_2 = lean_ctor_get_uint8(x_1, sizeof(void*)*4); +x_2 = lean_ctor_get_uint8(x_1, sizeof(void*)*5); x_3 = lean_box(x_2); if (lean_obj_tag(x_3) == 3) { @@ -2190,1654 +2483,1296 @@ x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_defaultCtorName___clo return x_1; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; -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_is_exclusive(x_12); -if (x_13 == 0) +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; lean_object* x_17; +x_12 = lean_unsigned_to_nat(1u); +x_13 = l_Lean_Syntax_getArg(x_1, x_12); +x_14 = l_Lean_Syntax_getId(x_13); +lean_inc(x_14); +x_15 = l_Lean_Name_append(x_2, x_14); +x_16 = lean_ctor_get_uint8(x_3, sizeof(void*)*3); +lean_inc(x_5); +x_17 = l_Lean_Elab_applyVisibility___at_Lean_Elab_Term_expandDeclId___spec__5(x_16, x_15, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_17) == 0) { -lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; -x_14 = lean_ctor_get(x_12, 0); -x_15 = lean_ctor_get(x_12, 1); -x_16 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(x_14, x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_15); -lean_dec(x_2); -x_17 = !lean_is_exclusive(x_16); -if (x_17 == 0) +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +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_3, 1); +lean_inc(x_20); +lean_inc(x_5); +lean_inc(x_18); +x_21 = l_Lean_addDocString_x27___at_Lean_Elab_Term_expandDeclId___spec__8(x_18, x_20, x_5, x_6, x_7, x_8, x_9, x_10, x_19); +if (lean_obj_tag(x_21) == 0) { -lean_object* x_18; -x_18 = lean_ctor_get(x_16, 0); -lean_ctor_set(x_12, 1, x_18); -lean_ctor_set(x_12, 0, x_11); -lean_ctor_set_tag(x_16, 1); -lean_ctor_set(x_16, 0, x_12); -return x_16; +lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; +x_22 = lean_ctor_get(x_21, 1); +lean_inc(x_22); +lean_dec(x_21); +x_23 = lean_box(0); +lean_inc(x_18); +x_24 = l_Lean_Elab_addDeclarationRangesFromSyntax___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3(x_18, x_13, x_23, x_5, x_6, x_7, x_8, x_9, x_10, x_22); +lean_dec(x_5); +x_25 = !lean_is_exclusive(x_24); +if (x_25 == 0) +{ +lean_object* x_26; lean_object* x_27; +x_26 = lean_ctor_get(x_24, 0); +lean_dec(x_26); +x_27 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_27, 0, x_13); +lean_ctor_set(x_27, 1, x_3); +lean_ctor_set(x_27, 2, x_14); +lean_ctor_set(x_27, 3, x_18); +lean_ctor_set(x_24, 0, x_27); +return x_24; } 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_12, 1, x_19); -lean_ctor_set(x_12, 0, x_11); -x_21 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_21, 0, x_12); -lean_ctor_set(x_21, 1, x_20); +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_alloc_ctor(0, 4, 0); +lean_ctor_set(x_29, 0, x_13); +lean_ctor_set(x_29, 1, x_3); +lean_ctor_set(x_29, 2, x_14); +lean_ctor_set(x_29, 3, x_18); +x_30 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_30, 0, x_29); +lean_ctor_set(x_30, 1, x_28); +return x_30; +} +} +else +{ +uint8_t x_31; +lean_dec(x_18); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_9); +lean_dec(x_5); +lean_dec(x_3); +x_31 = !lean_is_exclusive(x_21); +if (x_31 == 0) +{ return x_21; } +else +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_21, 0); +x_33 = lean_ctor_get(x_21, 1); +lean_inc(x_33); +lean_inc(x_32); +lean_dec(x_21); +x_34 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_34, 0, x_32); +lean_ctor_set(x_34, 1, x_33); +return x_34; +} +} } 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; -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 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(x_22, x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_23); -lean_dec(x_2); -x_25 = lean_ctor_get(x_24, 0); -lean_inc(x_25); -x_26 = lean_ctor_get(x_24, 1); -lean_inc(x_26); -if (lean_is_exclusive(x_24)) { - lean_ctor_release(x_24, 0); - lean_ctor_release(x_24, 1); - x_27 = x_24; -} else { - lean_dec_ref(x_24); - x_27 = lean_box(0); +uint8_t x_35; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_9); +lean_dec(x_5); +lean_dec(x_3); +x_35 = !lean_is_exclusive(x_17); +if (x_35 == 0) +{ +return x_17; } -x_28 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_28, 0, x_11); -lean_ctor_set(x_28, 1, x_25); -if (lean_is_scalar(x_27)) { - x_29 = lean_alloc_ctor(1, 2, 0); -} else { - x_29 = x_27; - lean_ctor_set_tag(x_29, 1); +else +{ +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_17, 0); +x_37 = lean_ctor_get(x_17, 1); +lean_inc(x_37); +lean_inc(x_36); +lean_dec(x_17); +x_38 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_38, 0, x_36); +lean_ctor_set(x_38, 1, x_37); +return x_38; } -lean_ctor_set(x_29, 0, x_28); -lean_ctor_set(x_29, 1, x_26); -return x_29; } } } -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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) { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__2___closed__1() { _start: { -uint8_t x_10; -x_10 = !lean_is_exclusive(x_7); -if (x_10 == 0) +lean_object* x_1; +x_1 = lean_mk_string_unchecked("invalid 'protected' constructor in a 'private' structure", 56, 56); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__2___closed__2() { +_start: { -lean_object* x_11; lean_object* x_12; lean_object* x_13; -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_Structure_0__Lean_Elab_Command_expandCtor___spec__7(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_7); -return x_13; +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__2___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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; +x_13 = l_Lean_Elab_Modifiers_isProtected(x_3); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; +x_14 = lean_box(0); +x_15 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__1(x_1, x_2, x_3, x_14, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +return x_15; } 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; uint8_t x_25; lean_object* x_26; uint8_t x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_14 = lean_ctor_get(x_7, 0); -x_15 = lean_ctor_get(x_7, 1); -x_16 = lean_ctor_get(x_7, 2); -x_17 = lean_ctor_get(x_7, 3); -x_18 = lean_ctor_get(x_7, 4); -x_19 = lean_ctor_get(x_7, 5); -x_20 = lean_ctor_get(x_7, 6); -x_21 = lean_ctor_get(x_7, 7); -x_22 = lean_ctor_get(x_7, 8); -x_23 = lean_ctor_get(x_7, 9); -x_24 = lean_ctor_get(x_7, 10); -x_25 = lean_ctor_get_uint8(x_7, sizeof(void*)*12); -x_26 = lean_ctor_get(x_7, 11); -x_27 = lean_ctor_get_uint8(x_7, sizeof(void*)*12 + 1); -lean_inc(x_26); -lean_inc(x_24); +uint8_t x_16; +x_16 = l_Lean_Elab_Modifiers_isPrivate(x_4); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; +x_17 = lean_box(0); +x_18 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__1(x_1, x_2, x_3, x_17, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +return x_18; +} +else +{ +lean_object* x_19; lean_object* x_20; uint8_t x_21; +lean_dec(x_3); +lean_dec(x_2); +x_19 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__2___closed__2; +x_20 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_19, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_10); +x_21 = !lean_is_exclusive(x_20); +if (x_21 == 0) +{ +return x_20; +} +else +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_20, 0); +x_23 = lean_ctor_get(x_20, 1); lean_inc(x_23); lean_inc(x_22); -lean_inc(x_21); -lean_inc(x_20); -lean_inc(x_19); -lean_inc(x_18); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_15); -lean_inc(x_14); -lean_dec(x_7); -x_28 = l_Lean_replaceRef(x_1, x_19); -lean_dec(x_19); -x_29 = lean_alloc_ctor(0, 12, 2); -lean_ctor_set(x_29, 0, x_14); -lean_ctor_set(x_29, 1, x_15); -lean_ctor_set(x_29, 2, x_16); -lean_ctor_set(x_29, 3, x_17); -lean_ctor_set(x_29, 4, x_18); -lean_ctor_set(x_29, 5, x_28); -lean_ctor_set(x_29, 6, x_20); -lean_ctor_set(x_29, 7, x_21); -lean_ctor_set(x_29, 8, x_22); -lean_ctor_set(x_29, 9, x_23); -lean_ctor_set(x_29, 10, x_24); -lean_ctor_set(x_29, 11, x_26); -lean_ctor_set_uint8(x_29, sizeof(void*)*12, x_25); -lean_ctor_set_uint8(x_29, sizeof(void*)*12 + 1, x_27); -x_30 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__7(x_2, x_3, x_4, x_5, x_6, x_29, x_8, x_9); -lean_dec(x_29); -return x_30; +lean_dec(x_20); +x_24 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); +return x_24; } } } -static lean_object* _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("runtime", 7, 7); -return x_1; } } -static lean_object* _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__2() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("maxRecDepth", 11, 11); +x_1 = lean_mk_string_unchecked("invalid 'private' constructor in a 'private' structure", 54, 54); return x_1; } } -static lean_object* _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__1; -x_2 = l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__2; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__4() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_maxRecDepthErrorMessage; -x_2 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_2, 0, x_1); +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__5() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__4; -x_2 = l_Lean_MessageData_ofFormat(x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__6() { -_start: +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_11 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_defaultCtorName; +lean_inc(x_3); +x_12 = l_Lean_Name_append(x_3, x_11); +x_13 = lean_unsigned_to_nat(1u); +x_14 = l_Lean_Syntax_getArg(x_1, x_13); +x_15 = l_Lean_Syntax_mkSynthetic(x_14); +x_16 = lean_unsigned_to_nat(5u); +x_17 = l_Lean_Syntax_getArg(x_1, x_16); +x_18 = l_Lean_Syntax_isNone(x_17); +if (x_18 == 0) { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__3; -x_2 = l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__5; -x_3 = lean_alloc_ctor(8, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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_19; uint8_t x_20; +x_19 = l_Lean_Syntax_getArg(x_17, x_13); +lean_dec(x_17); +x_20 = l_Lean_Syntax_isNone(x_19); +if (x_20 == 0) { -lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_9 = l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__6; -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_1); -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_8); -return x_11; -} -} -static lean_object* _init_l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__9___rarg___closed__1() { -_start: +lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; +lean_dec(x_15); +lean_dec(x_12); +x_21 = lean_unsigned_to_nat(0u); +x_22 = l_Lean_Syntax_getArg(x_19, x_21); +lean_dec(x_19); +x_23 = l_Lean_Syntax_getArg(x_22, x_21); +x_24 = !lean_is_exclusive(x_8); +if (x_24 == 0) { -lean_object* x_1; -x_1 = l_Lean_Elab_unsupportedSyntaxExceptionId; -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__9___rarg___closed__2() { -_start: +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_8, 5); +x_26 = l_Lean_replaceRef(x_22, x_25); +lean_dec(x_25); +lean_ctor_set(x_8, 5, x_26); +lean_inc(x_8); +lean_inc(x_4); +x_27 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6(x_23, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_27) == 0) { -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_Structure_0__Lean_Elab_Command_expandCtor___spec__9___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_Structure_0__Lean_Elab_Command_expandCtor___spec__9___rarg(lean_object* x_1) { -_start: +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_27, 0); +lean_inc(x_28); +x_29 = lean_ctor_get(x_27, 1); +lean_inc(x_29); +lean_dec(x_27); +lean_inc(x_4); +x_30 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__22(x_28, x_4, x_5, x_6, x_7, x_8, x_9, x_29); +if (lean_obj_tag(x_30) == 0) { -lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__9___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_Structure_0__Lean_Elab_Command_expandCtor___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) { -_start: +lean_object* x_31; uint8_t x_32; +x_31 = lean_ctor_get(x_30, 1); +lean_inc(x_31); +lean_dec(x_30); +x_32 = l_Lean_Elab_Modifiers_isPrivate(x_28); +if (x_32 == 0) { -lean_object* x_7; -x_7 = lean_alloc_closure((void*)(l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__9___rarg), 1, 0); -return x_7; -} +lean_object* x_33; lean_object* x_34; +x_33 = lean_box(0); +x_34 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__2(x_22, x_3, x_28, x_2, x_33, x_4, x_5, x_6, x_7, x_8, x_9, x_31); +lean_dec(x_22); +return x_34; } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__5___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; -x_5 = l_Lean_Elab_expandMacroImpl_x3f(x_1, x_2, x_3, x_4); -x_6 = lean_ctor_get(x_5, 0); -lean_inc(x_6); -if (lean_obj_tag(x_6) == 0) +uint8_t x_35; +x_35 = l_Lean_Elab_Modifiers_isPrivate(x_2); +if (x_35 == 0) { -uint8_t x_7; -x_7 = !lean_is_exclusive(x_5); -if (x_7 == 0) +lean_object* x_36; lean_object* x_37; +x_36 = lean_box(0); +x_37 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__2(x_22, x_3, x_28, x_2, x_36, x_4, x_5, x_6, x_7, x_8, x_9, x_31); +lean_dec(x_22); +return x_37; +} +else { -lean_object* x_8; lean_object* x_9; -x_8 = lean_ctor_get(x_5, 0); +lean_object* x_38; lean_object* x_39; uint8_t x_40; +lean_dec(x_28); +lean_dec(x_22); +lean_dec(x_3); +x_38 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__2; +x_39 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_38, x_4, x_5, x_6, x_7, x_8, x_9, x_31); lean_dec(x_8); -x_9 = lean_box(0); -lean_ctor_set(x_5, 0, x_9); -return x_5; +x_40 = !lean_is_exclusive(x_39); +if (x_40 == 0) +{ +return x_39; } else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_10 = lean_ctor_get(x_5, 1); -lean_inc(x_10); -lean_dec(x_5); -x_11 = lean_box(0); -x_12 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_12, 0, x_11); -lean_ctor_set(x_12, 1, x_10); -return x_12; +lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_41 = lean_ctor_get(x_39, 0); +x_42 = lean_ctor_get(x_39, 1); +lean_inc(x_42); +lean_inc(x_41); +lean_dec(x_39); +x_43 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_43, 0, x_41); +lean_ctor_set(x_43, 1, x_42); +return x_43; +} +} } } else { -uint8_t x_13; -x_13 = !lean_is_exclusive(x_6); -if (x_13 == 0) -{ -lean_object* x_14; lean_object* x_15; -x_14 = lean_ctor_get(x_6, 0); -x_15 = lean_ctor_get(x_14, 1); -lean_inc(x_15); -lean_dec(x_14); -if (lean_obj_tag(x_15) == 0) +uint8_t x_44; +lean_dec(x_28); +lean_dec(x_8); +lean_dec(x_22); +lean_dec(x_4); +lean_dec(x_3); +x_44 = !lean_is_exclusive(x_30); +if (x_44 == 0) { -lean_object* x_16; uint8_t x_17; -lean_free_object(x_6); -x_16 = lean_ctor_get(x_5, 1); -lean_inc(x_16); -lean_dec(x_5); -x_17 = !lean_is_exclusive(x_15); -if (x_17 == 0) -{ -lean_object* x_18; -x_18 = l_liftExcept___at_Lean_Elab_liftMacroM___spec__1(x_15, x_3, x_16); -lean_dec(x_15); -return x_18; +return x_30; } 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 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_20, 0, x_19); -x_21 = l_liftExcept___at_Lean_Elab_liftMacroM___spec__1(x_20, x_3, x_16); -lean_dec(x_20); -return x_21; +lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_45 = lean_ctor_get(x_30, 0); +x_46 = lean_ctor_get(x_30, 1); +lean_inc(x_46); +lean_inc(x_45); +lean_dec(x_30); +x_47 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_47, 0, x_45); +lean_ctor_set(x_47, 1, x_46); +return x_47; +} } } else { -lean_object* x_22; uint8_t x_23; -x_22 = lean_ctor_get(x_5, 1); -lean_inc(x_22); -lean_dec(x_5); -x_23 = !lean_is_exclusive(x_15); -if (x_23 == 0) +uint8_t x_48; +lean_dec(x_8); +lean_dec(x_22); +lean_dec(x_4); +lean_dec(x_3); +x_48 = !lean_is_exclusive(x_27); +if (x_48 == 0) { -lean_object* x_24; lean_object* x_25; -x_24 = lean_ctor_get(x_15, 0); -lean_ctor_set(x_6, 0, x_24); -lean_ctor_set(x_15, 0, x_6); -x_25 = l_liftExcept___at_Lean_Elab_liftMacroM___spec__1(x_15, x_3, x_22); -lean_dec(x_15); -return x_25; +return x_27; } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_15, 0); -lean_inc(x_26); -lean_dec(x_15); -lean_ctor_set(x_6, 0, x_26); -x_27 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_27, 0, x_6); -x_28 = l_liftExcept___at_Lean_Elab_liftMacroM___spec__1(x_27, x_3, x_22); +lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_49 = lean_ctor_get(x_27, 0); +x_50 = lean_ctor_get(x_27, 1); +lean_inc(x_50); +lean_inc(x_49); lean_dec(x_27); -return x_28; +x_51 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_51, 0, x_49); +lean_ctor_set(x_51, 1, x_50); +return x_51; } } } else { -lean_object* x_29; lean_object* x_30; -x_29 = lean_ctor_get(x_6, 0); -lean_inc(x_29); -lean_dec(x_6); -x_30 = lean_ctor_get(x_29, 1); -lean_inc(x_30); -lean_dec(x_29); -if (lean_obj_tag(x_30) == 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; uint8_t x_63; lean_object* x_64; uint8_t x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; +x_52 = lean_ctor_get(x_8, 0); +x_53 = lean_ctor_get(x_8, 1); +x_54 = lean_ctor_get(x_8, 2); +x_55 = lean_ctor_get(x_8, 3); +x_56 = lean_ctor_get(x_8, 4); +x_57 = lean_ctor_get(x_8, 5); +x_58 = lean_ctor_get(x_8, 6); +x_59 = lean_ctor_get(x_8, 7); +x_60 = lean_ctor_get(x_8, 8); +x_61 = lean_ctor_get(x_8, 9); +x_62 = lean_ctor_get(x_8, 10); +x_63 = lean_ctor_get_uint8(x_8, sizeof(void*)*12); +x_64 = lean_ctor_get(x_8, 11); +x_65 = lean_ctor_get_uint8(x_8, sizeof(void*)*12 + 1); +lean_inc(x_64); +lean_inc(x_62); +lean_inc(x_61); +lean_inc(x_60); +lean_inc(x_59); +lean_inc(x_58); +lean_inc(x_57); +lean_inc(x_56); +lean_inc(x_55); +lean_inc(x_54); +lean_inc(x_53); +lean_inc(x_52); +lean_dec(x_8); +x_66 = l_Lean_replaceRef(x_22, x_57); +lean_dec(x_57); +x_67 = lean_alloc_ctor(0, 12, 2); +lean_ctor_set(x_67, 0, x_52); +lean_ctor_set(x_67, 1, x_53); +lean_ctor_set(x_67, 2, x_54); +lean_ctor_set(x_67, 3, x_55); +lean_ctor_set(x_67, 4, x_56); +lean_ctor_set(x_67, 5, x_66); +lean_ctor_set(x_67, 6, x_58); +lean_ctor_set(x_67, 7, x_59); +lean_ctor_set(x_67, 8, x_60); +lean_ctor_set(x_67, 9, x_61); +lean_ctor_set(x_67, 10, x_62); +lean_ctor_set(x_67, 11, x_64); +lean_ctor_set_uint8(x_67, sizeof(void*)*12, x_63); +lean_ctor_set_uint8(x_67, sizeof(void*)*12 + 1, x_65); +lean_inc(x_67); +lean_inc(x_4); +x_68 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6(x_23, x_4, x_5, x_6, x_7, x_67, x_9, x_10); +if (lean_obj_tag(x_68) == 0) { -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_31 = lean_ctor_get(x_5, 1); -lean_inc(x_31); -lean_dec(x_5); -x_32 = lean_ctor_get(x_30, 0); -lean_inc(x_32); -if (lean_is_exclusive(x_30)) { - lean_ctor_release(x_30, 0); - x_33 = x_30; -} else { - lean_dec_ref(x_30); - x_33 = lean_box(0); -} -if (lean_is_scalar(x_33)) { - x_34 = lean_alloc_ctor(0, 1, 0); -} else { - x_34 = x_33; +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_4); +x_71 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__22(x_69, x_4, x_5, x_6, x_7, x_67, x_9, x_70); +if (lean_obj_tag(x_71) == 0) +{ +lean_object* x_72; uint8_t x_73; +x_72 = lean_ctor_get(x_71, 1); +lean_inc(x_72); +lean_dec(x_71); +x_73 = l_Lean_Elab_Modifiers_isPrivate(x_69); +if (x_73 == 0) +{ +lean_object* x_74; lean_object* x_75; +x_74 = lean_box(0); +x_75 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__2(x_22, x_3, x_69, x_2, x_74, x_4, x_5, x_6, x_7, x_67, x_9, x_72); +lean_dec(x_22); +return x_75; } -lean_ctor_set(x_34, 0, x_32); -x_35 = l_liftExcept___at_Lean_Elab_liftMacroM___spec__1(x_34, x_3, x_31); -lean_dec(x_34); -return x_35; +else +{ +uint8_t x_76; +x_76 = l_Lean_Elab_Modifiers_isPrivate(x_2); +if (x_76 == 0) +{ +lean_object* x_77; lean_object* x_78; +x_77 = lean_box(0); +x_78 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__2(x_22, x_3, x_69, x_2, x_77, x_4, x_5, x_6, x_7, x_67, x_9, x_72); +lean_dec(x_22); +return x_78; } 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_5, 1); -lean_inc(x_36); -lean_dec(x_5); -x_37 = lean_ctor_get(x_30, 0); -lean_inc(x_37); -if (lean_is_exclusive(x_30)) { - lean_ctor_release(x_30, 0); - x_38 = x_30; +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_69); +lean_dec(x_22); +lean_dec(x_3); +x_79 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__2; +x_80 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_79, x_4, x_5, x_6, x_7, x_67, x_9, x_72); +lean_dec(x_67); +x_81 = lean_ctor_get(x_80, 0); +lean_inc(x_81); +x_82 = lean_ctor_get(x_80, 1); +lean_inc(x_82); +if (lean_is_exclusive(x_80)) { + lean_ctor_release(x_80, 0); + lean_ctor_release(x_80, 1); + x_83 = x_80; } else { - lean_dec_ref(x_30); - x_38 = lean_box(0); + lean_dec_ref(x_80); + x_83 = lean_box(0); } -x_39 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_39, 0, x_37); -if (lean_is_scalar(x_38)) { - x_40 = lean_alloc_ctor(1, 1, 0); +if (lean_is_scalar(x_83)) { + x_84 = lean_alloc_ctor(1, 2, 0); } else { - x_40 = x_38; + x_84 = x_83; } -lean_ctor_set(x_40, 0, x_39); -x_41 = l_liftExcept___at_Lean_Elab_liftMacroM___spec__1(x_40, x_3, x_36); -lean_dec(x_40); -return x_41; +lean_ctor_set(x_84, 0, x_81); +lean_ctor_set(x_84, 1, x_82); +return x_84; } } } +else +{ +lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; +lean_dec(x_69); +lean_dec(x_67); +lean_dec(x_22); +lean_dec(x_4); +lean_dec(x_3); +x_85 = lean_ctor_get(x_71, 0); +lean_inc(x_85); +x_86 = lean_ctor_get(x_71, 1); +lean_inc(x_86); +if (lean_is_exclusive(x_71)) { + lean_ctor_release(x_71, 0); + lean_ctor_release(x_71, 1); + x_87 = x_71; +} else { + lean_dec_ref(x_71); + x_87 = lean_box(0); } +if (lean_is_scalar(x_87)) { + x_88 = lean_alloc_ctor(1, 2, 0); +} else { + x_88 = x_87; } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__5___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; -x_5 = l_Lean_Environment_contains(x_1, x_2); -x_6 = lean_box(x_5); -x_7 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_7, 0, x_6); -lean_ctor_set(x_7, 1, x_4); -return x_7; +lean_ctor_set(x_88, 0, x_85); +lean_ctor_set(x_88, 1, x_86); +return x_88; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__5___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; -x_7 = l_Lean_ResolveName_resolveNamespace(x_1, x_2, x_3, 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_6); -return x_8; +lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; +lean_dec(x_67); +lean_dec(x_22); +lean_dec(x_4); +lean_dec(x_3); +x_89 = lean_ctor_get(x_68, 0); +lean_inc(x_89); +x_90 = lean_ctor_get(x_68, 1); +lean_inc(x_90); +if (lean_is_exclusive(x_68)) { + lean_ctor_release(x_68, 0); + lean_ctor_release(x_68, 1); + x_91 = x_68; +} else { + lean_dec_ref(x_68); + x_91 = lean_box(0); +} +if (lean_is_scalar(x_91)) { + x_92 = lean_alloc_ctor(1, 2, 0); +} else { + x_92 = x_91; } +lean_ctor_set(x_92, 0, x_89); +lean_ctor_set(x_92, 1, x_90); +return x_92; } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__5___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; -x_7 = l_Lean_ResolveName_resolveGlobalName(x_1, x_2, x_3, 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_6); -return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: +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; 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_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, 0); -lean_inc(x_12); -lean_dec(x_10); -x_13 = lean_ctor_get(x_6, 3); -lean_inc(x_13); -x_14 = lean_ctor_get(x_6, 4); -lean_inc(x_14); -x_15 = lean_ctor_get(x_6, 5); -lean_inc(x_15); -x_16 = lean_ctor_get(x_6, 6); -lean_inc(x_16); -x_17 = lean_ctor_get(x_6, 7); -lean_inc(x_17); -x_18 = lean_ctor_get(x_6, 10); -lean_inc(x_18); -lean_inc(x_12); -x_19 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__5___lambda__1___boxed), 4, 1); -lean_closure_set(x_19, 0, x_12); -lean_inc(x_16); -x_20 = lean_alloc_closure((void*)(l_ReaderT_pure___at_Lean_Elab_liftMacroM___spec__2___rarg___boxed), 3, 1); -lean_closure_set(x_20, 0, x_16); -lean_inc(x_12); -x_21 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__5___lambda__2___boxed), 4, 1); -lean_closure_set(x_21, 0, x_12); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_12); -x_22 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__5___lambda__3___boxed), 6, 3); -lean_closure_set(x_22, 0, x_12); -lean_closure_set(x_22, 1, x_16); -lean_closure_set(x_22, 2, x_17); +lean_object* x_93; lean_object* x_94; uint8_t x_95; +lean_dec(x_19); +lean_dec(x_3); +x_93 = lean_box(0); lean_inc(x_12); -x_23 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__5___lambda__4___boxed), 6, 3); -lean_closure_set(x_23, 0, x_12); -lean_closure_set(x_23, 1, x_16); -lean_closure_set(x_23, 2, x_17); -x_24 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_24, 0, x_19); -lean_ctor_set(x_24, 1, x_20); -lean_ctor_set(x_24, 2, x_21); -lean_ctor_set(x_24, 3, x_22); -lean_ctor_set(x_24, 4, x_23); -x_25 = lean_st_ref_get(x_7, x_11); -x_26 = !lean_is_exclusive(x_25); -if (x_26 == 0) -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_27 = lean_ctor_get(x_25, 0); -x_28 = lean_ctor_get(x_25, 1); -x_29 = lean_ctor_get(x_27, 1); -lean_inc(x_29); -lean_dec(x_27); -x_30 = lean_environment_main_module(x_12); -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_18); -lean_ctor_set(x_31, 3, x_13); -lean_ctor_set(x_31, 4, x_14); -lean_ctor_set(x_31, 5, x_15); -x_32 = lean_box(0); -lean_ctor_set(x_25, 1, x_32); -lean_ctor_set(x_25, 0, x_29); -x_33 = lean_apply_2(x_1, x_31, x_25); -if (lean_obj_tag(x_33) == 0) -{ -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t 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_ctor_get(x_35, 0); -lean_inc(x_36); -x_37 = lean_st_ref_take(x_7, x_28); -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_is_exclusive(x_38); -if (x_40 == 0) -{ -lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; -x_41 = lean_ctor_get(x_38, 1); -lean_dec(x_41); -lean_ctor_set(x_38, 1, x_36); -x_42 = lean_st_ref_set(x_7, x_38, x_39); -x_43 = lean_ctor_get(x_42, 1); -lean_inc(x_43); -lean_dec(x_42); -x_44 = lean_ctor_get(x_35, 1); -lean_inc(x_44); -lean_dec(x_35); -x_45 = l_List_reverse___rarg(x_44); -x_46 = l_List_forM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__2(x_45, x_2, x_3, x_4, x_5, x_6, x_7, x_43); -lean_dec(x_6); -lean_dec(x_2); -x_47 = !lean_is_exclusive(x_46); -if (x_47 == 0) -{ -lean_object* x_48; -x_48 = lean_ctor_get(x_46, 0); -lean_dec(x_48); -lean_ctor_set(x_46, 0, x_34); -return x_46; -} -else +x_94 = l_Lean_Elab_addDeclarationRangesFromSyntax___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3(x_12, x_15, x_93, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_4); +x_95 = !lean_is_exclusive(x_94); +if (x_95 == 0) { -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 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_50, 0, x_34); -lean_ctor_set(x_50, 1, x_49); -return x_50; -} +lean_object* x_96; lean_object* x_97; lean_object* x_98; +x_96 = lean_ctor_get(x_94, 0); +lean_dec(x_96); +x_97 = l_Lean_Elab_Command_instInhabitedStructCtorView___closed__2; +x_98 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_98, 0, x_15); +lean_ctor_set(x_98, 1, x_97); +lean_ctor_set(x_98, 2, x_11); +lean_ctor_set(x_98, 3, x_12); +lean_ctor_set(x_94, 0, x_98); +return x_94; } else { -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; -x_51 = lean_ctor_get(x_38, 0); -x_52 = lean_ctor_get(x_38, 2); -x_53 = lean_ctor_get(x_38, 3); -x_54 = lean_ctor_get(x_38, 4); -x_55 = lean_ctor_get(x_38, 5); -x_56 = lean_ctor_get(x_38, 6); -lean_inc(x_56); -lean_inc(x_55); -lean_inc(x_54); -lean_inc(x_53); -lean_inc(x_52); -lean_inc(x_51); -lean_dec(x_38); -x_57 = lean_alloc_ctor(0, 7, 0); -lean_ctor_set(x_57, 0, x_51); -lean_ctor_set(x_57, 1, x_36); -lean_ctor_set(x_57, 2, x_52); -lean_ctor_set(x_57, 3, x_53); -lean_ctor_set(x_57, 4, x_54); -lean_ctor_set(x_57, 5, x_55); -lean_ctor_set(x_57, 6, x_56); -x_58 = lean_st_ref_set(x_7, x_57, x_39); -x_59 = lean_ctor_get(x_58, 1); -lean_inc(x_59); -lean_dec(x_58); -x_60 = lean_ctor_get(x_35, 1); -lean_inc(x_60); -lean_dec(x_35); -x_61 = l_List_reverse___rarg(x_60); -x_62 = l_List_forM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__2(x_61, x_2, x_3, x_4, x_5, x_6, x_7, x_59); -lean_dec(x_6); -lean_dec(x_2); -x_63 = lean_ctor_get(x_62, 1); -lean_inc(x_63); -if (lean_is_exclusive(x_62)) { - lean_ctor_release(x_62, 0); - lean_ctor_release(x_62, 1); - x_64 = x_62; -} else { - lean_dec_ref(x_62); - x_64 = lean_box(0); -} -if (lean_is_scalar(x_64)) { - x_65 = lean_alloc_ctor(0, 2, 0); -} else { - x_65 = x_64; +lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; +x_99 = lean_ctor_get(x_94, 1); +lean_inc(x_99); +lean_dec(x_94); +x_100 = l_Lean_Elab_Command_instInhabitedStructCtorView___closed__2; +x_101 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_101, 0, x_15); +lean_ctor_set(x_101, 1, x_100); +lean_ctor_set(x_101, 2, x_11); +lean_ctor_set(x_101, 3, x_12); +x_102 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_102, 0, x_101); +lean_ctor_set(x_102, 1, x_99); +return x_102; } -lean_ctor_set(x_65, 0, x_34); -lean_ctor_set(x_65, 1, x_63); -return x_65; } } else { -lean_object* x_66; -x_66 = lean_ctor_get(x_33, 0); -lean_inc(x_66); -lean_dec(x_33); -if (lean_obj_tag(x_66) == 0) -{ -lean_object* x_67; lean_object* x_68; lean_object* x_69; uint8_t x_70; -x_67 = lean_ctor_get(x_66, 0); -lean_inc(x_67); -x_68 = lean_ctor_get(x_66, 1); -lean_inc(x_68); -lean_dec(x_66); -x_69 = l_Lean_maxRecDepthErrorMessage; -x_70 = lean_string_dec_eq(x_68, x_69); -if (x_70 == 0) +lean_object* x_103; lean_object* x_104; uint8_t x_105; +lean_dec(x_17); +lean_dec(x_3); +x_103 = lean_box(0); +lean_inc(x_12); +x_104 = l_Lean_Elab_addDeclarationRangesFromSyntax___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3(x_12, x_15, x_103, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_4); +x_105 = !lean_is_exclusive(x_104); +if (x_105 == 0) { -lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_71 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_71, 0, x_68); -x_72 = l_Lean_MessageData_ofFormat(x_71); -x_73 = l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__6(x_67, x_72, x_2, x_3, x_4, x_5, x_6, x_7, x_28); -lean_dec(x_67); -return x_73; +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 = l_Lean_Elab_Command_instInhabitedStructCtorView___closed__2; +x_108 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_108, 0, x_15); +lean_ctor_set(x_108, 1, x_107); +lean_ctor_set(x_108, 2, x_11); +lean_ctor_set(x_108, 3, x_12); +lean_ctor_set(x_104, 0, x_108); +return x_104; } else { -lean_object* x_74; -lean_dec(x_68); -x_74 = l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8(x_67, x_2, x_3, x_4, x_5, x_6, x_7, x_28); -lean_dec(x_6); -lean_dec(x_2); -return x_74; -} +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 = l_Lean_Elab_Command_instInhabitedStructCtorView___closed__2; +x_111 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_111, 0, x_15); +lean_ctor_set(x_111, 1, x_110); +lean_ctor_set(x_111, 2, x_11); +lean_ctor_set(x_111, 3, x_12); +x_112 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_112, 0, x_111); +lean_ctor_set(x_112, 1, x_109); +return x_112; } -else -{ -lean_object* x_75; -lean_dec(x_6); -lean_dec(x_2); -x_75 = l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__9___rarg(x_28); -return x_75; } } } -else +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, 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_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_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_ctor_get(x_76, 1); -lean_inc(x_78); -lean_dec(x_76); -x_79 = lean_environment_main_module(x_12); -x_80 = lean_alloc_ctor(0, 6, 0); -lean_ctor_set(x_80, 0, x_24); -lean_ctor_set(x_80, 1, x_79); -lean_ctor_set(x_80, 2, x_18); -lean_ctor_set(x_80, 3, x_13); -lean_ctor_set(x_80, 4, x_14); -lean_ctor_set(x_80, 5, x_15); -x_81 = lean_box(0); -x_82 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_82, 0, x_78); -lean_ctor_set(x_82, 1, x_81); -x_83 = lean_apply_2(x_1, x_80, x_82); -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_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; -x_84 = lean_ctor_get(x_83, 0); -lean_inc(x_84); -x_85 = lean_ctor_get(x_83, 1); -lean_inc(x_85); -lean_dec(x_83); -x_86 = lean_ctor_get(x_85, 0); -lean_inc(x_86); -x_87 = lean_st_ref_take(x_7, x_77); -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); -x_90 = lean_ctor_get(x_88, 0); -lean_inc(x_90); -x_91 = lean_ctor_get(x_88, 2); -lean_inc(x_91); -x_92 = lean_ctor_get(x_88, 3); -lean_inc(x_92); -x_93 = lean_ctor_get(x_88, 4); -lean_inc(x_93); -x_94 = lean_ctor_get(x_88, 5); -lean_inc(x_94); -x_95 = lean_ctor_get(x_88, 6); -lean_inc(x_95); -if (lean_is_exclusive(x_88)) { - lean_ctor_release(x_88, 0); - lean_ctor_release(x_88, 1); - lean_ctor_release(x_88, 2); - lean_ctor_release(x_88, 3); - lean_ctor_release(x_88, 4); - lean_ctor_release(x_88, 5); - lean_ctor_release(x_88, 6); - x_96 = x_88; -} else { - lean_dec_ref(x_88); - x_96 = lean_box(0); -} -if (lean_is_scalar(x_96)) { - x_97 = lean_alloc_ctor(0, 7, 0); -} else { - x_97 = x_96; -} -lean_ctor_set(x_97, 0, x_90); -lean_ctor_set(x_97, 1, x_86); -lean_ctor_set(x_97, 2, x_91); -lean_ctor_set(x_97, 3, x_92); -lean_ctor_set(x_97, 4, x_93); -lean_ctor_set(x_97, 5, x_94); -lean_ctor_set(x_97, 6, x_95); -x_98 = lean_st_ref_set(x_7, x_97, x_89); -x_99 = lean_ctor_get(x_98, 1); -lean_inc(x_99); -lean_dec(x_98); -x_100 = lean_ctor_get(x_85, 1); -lean_inc(x_100); -lean_dec(x_85); -x_101 = l_List_reverse___rarg(x_100); -x_102 = l_List_forM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__2(x_101, x_2, x_3, x_4, x_5, x_6, x_7, x_99); +lean_object* x_12; +x_12 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); -lean_dec(x_2); -x_103 = lean_ctor_get(x_102, 1); -lean_inc(x_103); -if (lean_is_exclusive(x_102)) { - lean_ctor_release(x_102, 0); - lean_ctor_release(x_102, 1); - x_104 = x_102; -} else { - lean_dec_ref(x_102); - x_104 = lean_box(0); -} -if (lean_is_scalar(x_104)) { - x_105 = lean_alloc_ctor(0, 2, 0); -} else { - x_105 = x_104; +lean_dec(x_4); +lean_dec(x_1); +return x_12; } -lean_ctor_set(x_105, 0, x_84); -lean_ctor_set(x_105, 1, x_103); -return x_105; } -else -{ -lean_object* x_106; -x_106 = lean_ctor_get(x_83, 0); -lean_inc(x_106); -lean_dec(x_83); -if (lean_obj_tag(x_106) == 0) +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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_107; lean_object* x_108; lean_object* x_109; uint8_t x_110; -x_107 = lean_ctor_get(x_106, 0); -lean_inc(x_107); -x_108 = lean_ctor_get(x_106, 1); -lean_inc(x_108); -lean_dec(x_106); -x_109 = l_Lean_maxRecDepthErrorMessage; -x_110 = lean_string_dec_eq(x_108, x_109); -if (x_110 == 0) -{ -lean_object* x_111; lean_object* x_112; lean_object* x_113; -x_111 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_111, 0, x_108); -x_112 = l_Lean_MessageData_ofFormat(x_111); -x_113 = l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__6(x_107, x_112, x_2, x_3, x_4, x_5, x_6, x_7, x_77); -lean_dec(x_107); -return x_113; +lean_object* x_13; +x_13 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_11); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_1); +return x_13; } -else +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: { -lean_object* x_114; -lean_dec(x_108); -x_114 = l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8(x_107, x_2, x_3, x_4, x_5, x_6, x_7, x_77); +lean_object* x_11; +x_11 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_7); lean_dec(x_6); +lean_dec(x_5); lean_dec(x_2); -return x_114; +lean_dec(x_1); +return x_11; } } -else +static lean_object* _init_l_Lean_Elab_Command_checkValidFieldModifier___lambda__1___closed__1() { +_start: { -lean_object* x_115; -lean_dec(x_6); -lean_dec(x_2); -x_115 = l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__9___rarg(x_77); -return x_115; -} +lean_object* x_1; +x_1 = lean_mk_string_unchecked("invalid use of attributes in field declaration", 46, 46); +return x_1; } } +static lean_object* _init_l_Lean_Elab_Command_checkValidFieldModifier___lambda__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_checkValidFieldModifier___lambda__1___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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_Lean_Elab_Command_checkValidFieldModifier___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_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; -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_is_exclusive(x_12); +lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_10 = lean_ctor_get(x_1, 2); +x_11 = lean_array_get_size(x_10); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_nat_dec_eq(x_11, x_12); +lean_dec(x_11); if (x_13 == 0) { -lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; -x_14 = lean_ctor_get(x_12, 0); -x_15 = lean_ctor_get(x_12, 1); -x_16 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(x_14, x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_15); -lean_dec(x_2); -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_12, 1, x_18); -lean_ctor_set(x_12, 0, x_11); -lean_ctor_set_tag(x_16, 1); -lean_ctor_set(x_16, 0, x_12); -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_12, 1, x_19); -lean_ctor_set(x_12, 0, x_11); -x_21 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_21, 0, x_12); -lean_ctor_set(x_21, 1, x_20); -return x_21; -} +lean_object* x_14; lean_object* x_15; +x_14 = l_Lean_Elab_Command_checkValidFieldModifier___lambda__1___closed__2; +x_15 = l_Lean_throwError___at_Lean_Elab_Term_throwErrorIfErrors___spec__1(x_14, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_15; } 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; -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 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(x_22, x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_23); -lean_dec(x_2); -x_25 = lean_ctor_get(x_24, 0); -lean_inc(x_25); -x_26 = lean_ctor_get(x_24, 1); -lean_inc(x_26); -if (lean_is_exclusive(x_24)) { - lean_ctor_release(x_24, 0); - lean_ctor_release(x_24, 1); - x_27 = x_24; -} else { - lean_dec_ref(x_24); - x_27 = lean_box(0); -} -x_28 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_28, 0, x_11); -lean_ctor_set(x_28, 1, x_25); -if (lean_is_scalar(x_27)) { - x_29 = lean_alloc_ctor(1, 2, 0); -} else { - x_29 = x_27; - lean_ctor_set_tag(x_29, 1); -} -lean_ctor_set(x_29, 0, x_28); -lean_ctor_set(x_29, 1, x_26); -return x_29; -} -} +lean_object* x_16; lean_object* x_17; +lean_dec(x_3); +x_16 = lean_box(0); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_16); +lean_ctor_set(x_17, 1, x_9); +return x_17; } -static lean_object* _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Lean", 4, 4); -return x_1; } } -static lean_object* _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__2() { +static lean_object* _init_l_Lean_Elab_Command_checkValidFieldModifier___lambda__2___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("Parser", 6, 6); +x_1 = lean_mk_string_unchecked("invalid use of 'unsafe' in field declaration", 44, 44); return x_1; } } -static lean_object* _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__3() { +static lean_object* _init_l_Lean_Elab_Command_checkValidFieldModifier___lambda__2___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Term", 4, 4); -return x_1; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_checkValidFieldModifier___lambda__2___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -static lean_object* _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__4() { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidFieldModifier___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("byTactic", 8, 8); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__5() { -_start: +uint8_t x_10; +x_10 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 3); +if (x_10 == 0) { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__1; -x_2 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__2; -x_3 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__3; -x_4 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__4; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; -} +lean_object* x_11; lean_object* x_12; +x_11 = lean_box(0); +x_12 = l_Lean_Elab_Command_checkValidFieldModifier___lambda__1(x_1, x_11, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_12; } -LEAN_EXPORT uint8_t l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1(lean_object* x_1) { -_start: +else { -lean_object* x_2; uint8_t x_3; -x_2 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__5; -x_3 = lean_name_eq(x_1, x_2); -if (x_3 == 0) +lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_13 = l_Lean_Elab_Command_checkValidFieldModifier___lambda__2___closed__2; +x_14 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 0) { -uint8_t x_4; -x_4 = 1; -return x_4; +return x_14; } else { -uint8_t x_5; -x_5 = 0; -return x_5; -} -} -} -static lean_object* _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("unknown attribute [", 19, 19); -return x_1; +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_14, 0); +x_17 = lean_ctor_get(x_14, 1); +lean_inc(x_17); +lean_inc(x_16); +lean_dec(x_14); +x_18 = lean_alloc_ctor(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_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; } } -static lean_object* _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2___closed__3() { +static lean_object* _init_l_Lean_Elab_Command_checkValidFieldModifier___lambda__3___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("]", 1, 1); +x_1 = lean_mk_string_unchecked("invalid use of 'partial' in field declaration", 45, 45); return x_1; } } -static lean_object* _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2___closed__4() { +static lean_object* _init_l_Lean_Elab_Command_checkValidFieldModifier___lambda__3___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2___closed__3; +x_1 = l_Lean_Elab_Command_checkValidFieldModifier___lambda__3___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___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, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidFieldModifier___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_11; uint8_t x_12; -x_11 = lean_st_ref_get(x_9, x_10); -x_12 = !lean_is_exclusive(x_11); -if (x_12 == 0) -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_13 = lean_ctor_get(x_11, 0); -x_14 = lean_ctor_get(x_11, 1); -x_15 = lean_ctor_get(x_13, 0); -lean_inc(x_15); -lean_dec(x_13); -lean_inc(x_3); -x_16 = l_Lean_getAttributeImpl(x_15, x_3); -lean_dec(x_15); -if (lean_obj_tag(x_16) == 0) -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -lean_dec(x_16); -lean_free_object(x_11); -lean_dec(x_2); -x_17 = l_Lean_MessageData_ofName(x_3); -x_18 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2___closed__2; -x_19 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_19, 0, x_18); -lean_ctor_set(x_19, 1, x_17); -x_20 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2___closed__4; -x_21 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_21, 0, x_19); -lean_ctor_set(x_21, 1, x_20); -x_22 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__10(x_21, x_4, x_5, x_6, x_7, x_8, x_9, x_14); -return x_22; -} -else +uint8_t x_10; +x_10 = l_Lean_Elab_Modifiers_isPartial(x_1); +if (x_10 == 0) { -lean_object* x_23; -lean_dec(x_16); -lean_dec(x_4); -x_23 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_23, 0, x_3); -lean_ctor_set(x_23, 1, x_2); -lean_ctor_set_uint8(x_23, sizeof(void*)*2, x_1); -lean_ctor_set(x_11, 0, x_23); -return x_11; -} +lean_object* x_11; lean_object* x_12; +x_11 = lean_box(0); +x_12 = l_Lean_Elab_Command_checkValidFieldModifier___lambda__2(x_1, x_11, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_12; } else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_24 = lean_ctor_get(x_11, 0); -x_25 = lean_ctor_get(x_11, 1); -lean_inc(x_25); -lean_inc(x_24); -lean_dec(x_11); -x_26 = lean_ctor_get(x_24, 0); -lean_inc(x_26); -lean_dec(x_24); -lean_inc(x_3); -x_27 = l_Lean_getAttributeImpl(x_26, x_3); -lean_dec(x_26); -if (lean_obj_tag(x_27) == 0) +lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_13 = l_Lean_Elab_Command_checkValidFieldModifier___lambda__3___closed__2; +x_14 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 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_dec(x_27); -lean_dec(x_2); -x_28 = l_Lean_MessageData_ofName(x_3); -x_29 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2___closed__2; -x_30 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_30, 0, x_29); -lean_ctor_set(x_30, 1, x_28); -x_31 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2___closed__4; -x_32 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_32, 0, x_30); -lean_ctor_set(x_32, 1, x_31); -x_33 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__10(x_32, x_4, x_5, x_6, x_7, x_8, x_9, x_25); -return x_33; +return x_14; } else { -lean_object* x_34; lean_object* x_35; -lean_dec(x_27); -lean_dec(x_4); -x_34 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_34, 0, x_3); -lean_ctor_set(x_34, 1, x_2); -lean_ctor_set_uint8(x_34, sizeof(void*)*2, x_1); -x_35 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_35, 0, x_34); -lean_ctor_set(x_35, 1, x_25); -return x_35; +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_14, 0); +x_17 = lean_ctor_get(x_14, 1); +lean_inc(x_17); +lean_inc(x_16); +lean_dec(x_14); +x_18 = lean_alloc_ctor(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_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__1() { +static lean_object* _init_l_Lean_Elab_Command_checkValidFieldModifier___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___boxed), 1, 0); +x_1 = lean_mk_string_unchecked("invalid use of 'noncomputable' in field declaration", 51, 51); return x_1; } } -static lean_object* _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__2() { +static lean_object* _init_l_Lean_Elab_Command_checkValidFieldModifier___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Attr", 4, 4); -return x_1; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_checkValidFieldModifier___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -static lean_object* _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__3() { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidFieldModifier(lean_object* x_1, lean_object* x_2, lean_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_unchecked("simple", 6, 6); -return x_1; -} +uint8_t x_9; +x_9 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 1); +if (x_9 == 0) +{ +lean_object* x_10; lean_object* x_11; +x_10 = lean_box(0); +x_11 = l_Lean_Elab_Command_checkValidFieldModifier___lambda__3(x_1, x_10, 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; uint8_t x_14; +x_12 = l_Lean_Elab_Command_checkValidFieldModifier___closed__2; +x_13 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_14 = !lean_is_exclusive(x_13); +if (x_14 == 0) +{ +return x_13; +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_15 = lean_ctor_get(x_13, 0); +x_16 = lean_ctor_get(x_13, 1); +lean_inc(x_16); +lean_inc(x_15); +lean_dec(x_13); +x_17 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_17, 0, x_15); +lean_ctor_set(x_17, 1, x_16); +return x_17; +} +} } -static lean_object* _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__4() { +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidFieldModifier___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, 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; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__1; -x_2 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__2; -x_3 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__2; -x_4 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__3; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; +lean_object* x_10; +x_10 = l_Lean_Elab_Command_checkValidFieldModifier___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +return x_10; } } -static lean_object* _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__5() { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidFieldModifier___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_1; -x_1 = lean_mk_string_unchecked("unknown attribute", 17, 17); -return x_1; +lean_object* x_10; +x_10 = l_Lean_Elab_Command_checkValidFieldModifier___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +return x_10; } } -static lean_object* _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__6() { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidFieldModifier___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__5; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +lean_object* x_10; +x_10 = l_Lean_Elab_Command_checkValidFieldModifier___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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_EXPORT lean_object* l_Lean_Elab_Command_checkValidFieldModifier___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_9 = lean_unsigned_to_nat(0u); -x_10 = l_Lean_Syntax_getArg(x_1, x_9); -x_11 = lean_alloc_closure((void*)(l_Lean_Elab_toAttributeKind___boxed), 3, 1); -lean_closure_set(x_11, 0, x_10); -lean_inc(x_6); -lean_inc(x_2); -x_12 = l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__5(x_11, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_12) == 0) +lean_object* x_9; +x_9 = l_Lean_Elab_Command_checkValidFieldModifier(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); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___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_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18) { +_start: { -lean_object* x_13; 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_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_unsigned_to_nat(1u); -x_16 = l_Lean_Syntax_getArg(x_1, x_15); -x_17 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__1; -x_18 = lean_alloc_closure((void*)(l_Lean_expandMacros), 4, 2); -lean_closure_set(x_18, 0, x_16); -lean_closure_set(x_18, 1, x_17); -lean_inc(x_6); +lean_object* x_19; uint8_t x_20; lean_object* x_21; lean_inc(x_2); -x_19 = l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__9(x_18, x_2, x_3, x_4, x_5, x_6, x_7, x_14); -if (lean_obj_tag(x_19) == 0) -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_19, 1); -lean_inc(x_21); -lean_dec(x_19); -lean_inc(x_20); -x_22 = l_Lean_Syntax_getKind(x_20); -x_23 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__4; -x_24 = lean_name_eq(x_22, x_23); -if (x_24 == 0) -{ -if (lean_obj_tag(x_22) == 1) +x_19 = l_Lean_Name_append(x_1, x_2); +x_20 = lean_ctor_get_uint8(x_3, sizeof(void*)*3); +lean_inc(x_12); +x_21 = l_Lean_Elab_applyVisibility___at_Lean_Elab_Term_expandDeclId___spec__5(x_20, x_19, x_12, x_13, x_14, x_15, x_16, x_17, x_18); +if (lean_obj_tag(x_21) == 0) { -lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; lean_object* x_29; -x_25 = lean_ctor_get(x_22, 1); -lean_inc(x_25); -lean_dec(x_22); -x_26 = lean_box(0); -x_27 = l_Lean_Name_str___override(x_26, x_25); -x_28 = lean_unbox(x_13); -lean_dec(x_13); -x_29 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2(x_28, x_20, x_27, x_2, x_3, x_4, x_5, x_6, x_7, x_21); -lean_dec(x_6); -return x_29; -} -else +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_ctor_get(x_3, 1); +lean_inc(x_24); +lean_inc(x_22); +x_25 = l_Lean_addDocString_x27___at_Lean_Elab_Term_expandDeclId___spec__8(x_22, x_24, x_12, x_13, x_14, x_15, x_16, x_17, x_23); +if (lean_obj_tag(x_25) == 0) { -lean_object* x_30; lean_object* x_31; uint8_t x_32; -lean_dec(x_22); -lean_dec(x_13); -x_30 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__6; -x_31 = l_Lean_throwErrorAt___at_Lean_Elab_Term_processDefDeriving___spec__2(x_20, x_30, x_2, x_3, x_4, x_5, x_6, x_7, x_21); -lean_dec(x_20); -x_32 = !lean_is_exclusive(x_31); -if (x_32 == 0) +uint8_t x_26; +x_26 = !lean_is_exclusive(x_25); +if (x_26 == 0) { -return x_31; +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_25, 0); +lean_dec(x_27); +lean_inc(x_4); +x_28 = lean_alloc_ctor(0, 9, 1); +lean_ctor_set(x_28, 0, x_4); +lean_ctor_set(x_28, 1, x_3); +lean_ctor_set(x_28, 2, x_22); +lean_ctor_set(x_28, 3, x_4); +lean_ctor_set(x_28, 4, x_2); +lean_ctor_set(x_28, 5, x_6); +lean_ctor_set(x_28, 6, x_7); +lean_ctor_set(x_28, 7, x_8); +lean_ctor_set(x_28, 8, x_9); +lean_ctor_set_uint8(x_28, sizeof(void*)*9, x_5); +x_29 = lean_array_push(x_10, x_28); +lean_ctor_set(x_25, 0, x_29); +return x_25; } else { -lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_33 = lean_ctor_get(x_31, 0); -x_34 = lean_ctor_get(x_31, 1); -lean_inc(x_34); -lean_inc(x_33); -lean_dec(x_31); -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_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_30 = lean_ctor_get(x_25, 1); +lean_inc(x_30); +lean_dec(x_25); +lean_inc(x_4); +x_31 = lean_alloc_ctor(0, 9, 1); +lean_ctor_set(x_31, 0, x_4); +lean_ctor_set(x_31, 1, x_3); +lean_ctor_set(x_31, 2, x_22); +lean_ctor_set(x_31, 3, x_4); +lean_ctor_set(x_31, 4, x_2); +lean_ctor_set(x_31, 5, x_6); +lean_ctor_set(x_31, 6, x_7); +lean_ctor_set(x_31, 7, x_8); +lean_ctor_set(x_31, 8, x_9); +lean_ctor_set_uint8(x_31, sizeof(void*)*9, x_5); +x_32 = lean_array_push(x_10, x_31); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_30); +return x_33; } } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; lean_object* x_40; +uint8_t x_34; lean_dec(x_22); -x_36 = l_Lean_Syntax_getArg(x_20, x_9); -x_37 = l_Lean_Syntax_getId(x_36); -lean_dec(x_36); -x_38 = lean_erase_macro_scopes(x_37); -x_39 = lean_unbox(x_13); -lean_dec(x_13); -x_40 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2(x_39, x_20, x_38, x_2, x_3, x_4, x_5, x_6, x_7, x_21); -lean_dec(x_6); -return x_40; -} -} -else -{ -uint8_t x_41; -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_4); +lean_dec(x_3); lean_dec(x_2); -x_41 = !lean_is_exclusive(x_19); -if (x_41 == 0) +x_34 = !lean_is_exclusive(x_25); +if (x_34 == 0) { -return x_19; +return x_25; } else { -lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_ctor_get(x_19, 0); -x_43 = lean_ctor_get(x_19, 1); -lean_inc(x_43); -lean_inc(x_42); -lean_dec(x_19); -x_44 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_44, 0, x_42); -lean_ctor_set(x_44, 1, x_43); -return x_44; +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_25, 0); +x_36 = lean_ctor_get(x_25, 1); +lean_inc(x_36); +lean_inc(x_35); +lean_dec(x_25); +x_37 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +return x_37; } } } else { -uint8_t x_45; +uint8_t x_38; +lean_dec(x_12); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); +lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); -x_45 = !lean_is_exclusive(x_12); -if (x_45 == 0) +x_38 = !lean_is_exclusive(x_21); +if (x_38 == 0) { -return x_12; +return x_21; } else { -lean_object* x_46; lean_object* x_47; lean_object* x_48; -x_46 = lean_ctor_get(x_12, 0); -x_47 = lean_ctor_get(x_12, 1); -lean_inc(x_47); -lean_inc(x_46); -lean_dec(x_12); -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_39; lean_object* x_40; lean_object* x_41; +x_39 = lean_ctor_get(x_21, 0); +x_40 = lean_ctor_get(x_21, 1); +lean_inc(x_40); +lean_inc(x_39); +lean_dec(x_21); +x_41 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_41, 0, x_39); +lean_ctor_set(x_41, 1, x_40); +return x_41; } } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__11(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) { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___closed__1() { _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_9); -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; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("invalid field name '", 20, 20); +return x_1; } -else +} +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___closed__2() { +_start: { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; lean_object* x_27; uint8_t x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; -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_object* x_1; lean_object* x_2; +x_1 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("', field names must be atomic", 29, 29); +return x_1; +} +} +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___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, size_t x_8, size_t x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { +_start: +{ +uint8_t x_18; +x_18 = lean_usize_dec_eq(x_8, x_9); +if (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; 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; uint8_t x_36; lean_object* x_37; lean_object* x_38; +x_19 = lean_array_uget(x_7, x_8); +x_20 = l_Lean_Syntax_getId(x_19); 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 = lean_ctor_get_uint8(x_9, sizeof(void*)*12); -x_27 = lean_ctor_get(x_9, 11); +x_21 = lean_erase_macro_scopes(x_20); +x_22 = l_Lean_Name_isAtomic(x_21); +x_23 = lean_ctor_get(x_15, 0); +x_24 = lean_ctor_get(x_15, 1); +x_25 = lean_ctor_get(x_15, 2); +x_26 = lean_ctor_get(x_15, 3); +x_27 = lean_ctor_get(x_15, 4); +x_28 = lean_ctor_get(x_15, 5); +x_29 = lean_ctor_get(x_15, 6); +x_30 = lean_ctor_get(x_15, 7); +x_31 = lean_ctor_get(x_15, 8); +x_32 = lean_ctor_get(x_15, 9); +x_33 = lean_ctor_get(x_15, 10); +x_34 = lean_ctor_get_uint8(x_15, sizeof(void*)*12); +x_35 = lean_ctor_get(x_15, 11); +x_36 = lean_ctor_get_uint8(x_15, sizeof(void*)*12 + 1); +x_37 = l_Lean_replaceRef(x_19, x_28); +lean_inc(x_35); +lean_inc(x_33); +lean_inc(x_32); +lean_inc(x_31); +lean_inc(x_30); +lean_inc(x_29); lean_inc(x_27); -x_28 = lean_ctor_get_uint8(x_9, sizeof(void*)*12 + 1); -x_29 = l_Lean_replaceRef(x_14, x_20); +lean_inc(x_26); +lean_inc(x_25); +lean_inc(x_24); +lean_inc(x_23); +x_38 = lean_alloc_ctor(0, 12, 2); +lean_ctor_set(x_38, 0, x_23); +lean_ctor_set(x_38, 1, x_24); +lean_ctor_set(x_38, 2, x_25); +lean_ctor_set(x_38, 3, x_26); +lean_ctor_set(x_38, 4, x_27); +lean_ctor_set(x_38, 5, x_37); +lean_ctor_set(x_38, 6, x_29); +lean_ctor_set(x_38, 7, x_30); +lean_ctor_set(x_38, 8, x_31); +lean_ctor_set(x_38, 9, x_32); +lean_ctor_set(x_38, 10, x_33); +lean_ctor_set(x_38, 11, x_35); +lean_ctor_set_uint8(x_38, sizeof(void*)*12, x_34); +lean_ctor_set_uint8(x_38, sizeof(void*)*12 + 1, x_36); +if (x_22 == 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; uint8_t x_46; lean_dec(x_20); -x_30 = lean_alloc_ctor(0, 12, 2); -lean_ctor_set(x_30, 0, x_15); -lean_ctor_set(x_30, 1, x_16); -lean_ctor_set(x_30, 2, x_17); -lean_ctor_set(x_30, 3, x_18); -lean_ctor_set(x_30, 4, x_19); -lean_ctor_set(x_30, 5, x_29); -lean_ctor_set(x_30, 6, x_21); -lean_ctor_set(x_30, 7, x_22); -lean_ctor_set(x_30, 8, x_23); -lean_ctor_set(x_30, 9, x_24); -lean_ctor_set(x_30, 10, x_25); -lean_ctor_set(x_30, 11, x_27); -lean_ctor_set_uint8(x_30, sizeof(void*)*12, x_26); -lean_ctor_set_uint8(x_30, sizeof(void*)*12 + 1, x_28); -lean_inc(x_5); -x_31 = 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_30, x_10, x_11); -lean_dec(x_14); -if (lean_obj_tag(x_31) == 0) +lean_dec(x_10); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_39 = lean_erase_macro_scopes(x_21); +x_40 = l_Lean_MessageData_ofName(x_39); +x_41 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___closed__2; +x_42 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_42, 0, x_41); +lean_ctor_set(x_42, 1, x_40); +x_43 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___closed__4; +x_44 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_44, 0, x_42); +lean_ctor_set(x_44, 1, x_43); +x_45 = l_Lean_throwErrorAt___at___private_Lean_Elab_Binders_0__Lean_Elab_Term_elabBinderViews_loop___spec__1(x_19, x_44, x_11, x_12, x_13, x_14, x_38, x_16, x_17); +lean_dec(x_19); +x_46 = !lean_is_exclusive(x_45); +if (x_46 == 0) { -lean_object* x_32; lean_object* x_33; lean_object* x_34; size_t x_35; size_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_array_push(x_4, x_32); -x_35 = 1; -x_36 = lean_usize_add(x_3, x_35); -x_3 = x_36; -x_4 = x_34; -x_11 = x_33; -goto _start; +return x_45; } else { -uint8_t x_38; -x_38 = !lean_is_exclusive(x_31); -if (x_38 == 0) -{ -lean_object* x_39; lean_object* x_40; uint8_t x_41; -x_39 = lean_ctor_get(x_31, 0); -x_40 = lean_ctor_get(x_31, 1); -x_41 = l_Lean_Exception_isInterrupt(x_39); -if (x_41 == 0) -{ -uint8_t x_42; -x_42 = l_Lean_Exception_isRuntime(x_39); -if (x_42 == 0) +lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_47 = lean_ctor_get(x_45, 0); +x_48 = lean_ctor_get(x_45, 1); +lean_inc(x_48); +lean_inc(x_47); +lean_dec(x_45); +x_49 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_49, 0, x_47); +lean_ctor_set(x_49, 1, x_48); +return x_49; +} +} +else { -lean_object* x_43; -lean_free_object(x_31); -lean_inc(x_9); -x_43 = l_Lean_Elab_logException___at_Lean_Elab_Term_exceptionToSorry___spec__1(x_39, x_5, x_6, x_7, x_8, x_9, x_10, x_40); -if (lean_obj_tag(x_43) == 0) +lean_object* x_50; lean_object* x_51; +x_50 = lean_box(0); +lean_inc(x_11); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_1); +x_51 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___lambda__1(x_1, x_21, x_3, x_19, x_2, x_20, x_4, x_5, x_6, x_10, x_50, x_11, x_12, x_13, x_14, x_38, x_16, x_17); +lean_dec(x_38); +if (lean_obj_tag(x_51) == 0) { -lean_object* x_44; size_t x_45; size_t x_46; -x_44 = lean_ctor_get(x_43, 1); -lean_inc(x_44); -lean_dec(x_43); -x_45 = 1; -x_46 = lean_usize_add(x_3, x_45); -x_3 = x_46; -x_11 = x_44; +lean_object* x_52; lean_object* x_53; size_t x_54; size_t x_55; +x_52 = lean_ctor_get(x_51, 0); +lean_inc(x_52); +x_53 = lean_ctor_get(x_51, 1); +lean_inc(x_53); +lean_dec(x_51); +x_54 = 1; +x_55 = lean_usize_add(x_8, x_54); +x_8 = x_55; +x_10 = x_52; +x_17 = x_53; goto _start; } else { -uint8_t x_48; -lean_dec(x_9); +uint8_t x_57; +lean_dec(x_11); +lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_48 = !lean_is_exclusive(x_43); -if (x_48 == 0) +lean_dec(x_3); +lean_dec(x_1); +x_57 = !lean_is_exclusive(x_51); +if (x_57 == 0) { -return x_43; +return x_51; } 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_58; lean_object* x_59; lean_object* x_60; +x_58 = lean_ctor_get(x_51, 0); +x_59 = lean_ctor_get(x_51, 1); +lean_inc(x_59); +lean_inc(x_58); +lean_dec(x_51); +x_60 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_60, 0, x_58); +lean_ctor_set(x_60, 1, x_59); +return x_60; } } -else -{ -lean_dec(x_9); -lean_dec(x_5); -lean_dec(x_4); -return x_31; } } else { -lean_dec(x_9); +lean_object* x_61; +lean_dec(x_11); +lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -return x_31; +lean_dec(x_3); +lean_dec(x_1); +x_61 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_61, 0, x_10); +lean_ctor_set(x_61, 1, x_17); +return x_61; } } -else -{ -lean_object* x_52; lean_object* x_53; uint8_t x_54; -x_52 = lean_ctor_get(x_31, 0); -x_53 = lean_ctor_get(x_31, 1); -lean_inc(x_53); -lean_inc(x_52); -lean_dec(x_31); -x_54 = l_Lean_Exception_isInterrupt(x_52); -if (x_54 == 0) -{ -uint8_t x_55; -x_55 = l_Lean_Exception_isRuntime(x_52); -if (x_55 == 0) -{ -lean_object* x_56; -lean_inc(x_9); -x_56 = l_Lean_Elab_logException___at_Lean_Elab_Term_exceptionToSorry___spec__1(x_52, x_5, x_6, x_7, x_8, x_9, x_10, x_53); -if (lean_obj_tag(x_56) == 0) -{ -lean_object* x_57; size_t x_58; size_t x_59; -x_57 = lean_ctor_get(x_56, 1); -lean_inc(x_57); -lean_dec(x_56); -x_58 = 1; -x_59 = lean_usize_add(x_3, x_58); -x_3 = x_59; -x_11 = x_57; -goto _start; } -else -{ -lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; -lean_dec(x_9); -lean_dec(x_5); -lean_dec(x_4); -x_61 = lean_ctor_get(x_56, 0); -lean_inc(x_61); -x_62 = lean_ctor_get(x_56, 1); -lean_inc(x_62); -if (lean_is_exclusive(x_56)) { - lean_ctor_release(x_56, 0); - lean_ctor_release(x_56, 1); - x_63 = x_56; -} else { - lean_dec_ref(x_56); - x_63 = lean_box(0); -} -if (lean_is_scalar(x_63)) { - x_64 = lean_alloc_ctor(1, 2, 0); -} else { - x_64 = x_63; -} -lean_ctor_set(x_64, 0, x_61); -lean_ctor_set(x_64, 1, x_62); -return x_64; -} -} -else -{ -lean_object* x_65; -lean_dec(x_9); -lean_dec(x_5); -lean_dec(x_4); -x_65 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_65, 0, x_52); -lean_ctor_set(x_65, 1, x_53); -return x_65; -} -} -else -{ -lean_object* x_66; -lean_dec(x_9); -lean_dec(x_5); -lean_dec(x_4); -x_66 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_66, 0, x_52); -lean_ctor_set(x_66, 1, x_53); -return x_66; -} -} -} -} -} -} -static lean_object* _init_l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = lean_box(0); -x_2 = lean_array_mk(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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: -{ -size_t x_9; size_t x_10; lean_object* x_11; lean_object* x_12; -x_9 = lean_array_size(x_1); -x_10 = 0; -x_11 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; -x_12 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__11(x_1, x_9, x_10, x_11, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_12) == 0) -{ -uint8_t x_13; -x_13 = !lean_is_exclusive(x_12); -if (x_13 == 0) -{ -return x_12; -} -else -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_14 = lean_ctor_get(x_12, 0); -x_15 = lean_ctor_get(x_12, 1); -lean_inc(x_15); -lean_inc(x_14); -lean_dec(x_12); -x_16 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_16, 0, x_14); -lean_ctor_set(x_16, 1, x_15); -return x_16; -} -} -else -{ -uint8_t x_17; -x_17 = !lean_is_exclusive(x_12); -if (x_17 == 0) -{ -return x_12; -} -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_EXPORT lean_object* l_Lean_Elab_elabDeclAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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; -x_9 = lean_unsigned_to_nat(1u); -x_10 = l_Lean_Syntax_getArg(x_1, x_9); -x_11 = l_Lean_Syntax_getSepArgs(x_10); -lean_dec(x_10); -x_12 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3(x_11, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_11); -return x_12; -} -} -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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) { -_start: +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___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; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; x_9 = lean_ctor_get(x_6, 5); @@ -3918,7 +3853,7 @@ return x_29; } } } -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { uint8_t x_10; @@ -3930,7 +3865,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_Structure_0__Lean_Elab_Command_expandCtor___spec__13(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_13 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__3(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_7); return x_13; } @@ -3981,13 +3916,13 @@ lean_ctor_set(x_29, 10, x_24); lean_ctor_set(x_29, 11, x_26); lean_ctor_set_uint8(x_29, sizeof(void*)*12, x_25); lean_ctor_set_uint8(x_29, sizeof(void*)*12 + 1, x_27); -x_30 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__13(x_2, x_3, x_4, x_5, x_6, x_29, x_8, x_9); +x_30 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__3(x_2, x_3, x_4, x_5, x_6, x_29, x_8, x_9); lean_dec(x_29); return x_30; } } } -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; @@ -4069,2359 +4004,2658 @@ return x_29; } } } -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -uint8_t x_10; -x_10 = !lean_is_exclusive(x_7); -if (x_10 == 0) +lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_14 = lean_ctor_get(x_6, 1); +lean_inc(x_14); +x_15 = lean_ctor_get(x_6, 0); +lean_inc(x_15); +lean_dec(x_6); +x_16 = !lean_is_exclusive(x_14); +if (x_16 == 0) { -lean_object* x_11; lean_object* x_12; lean_object* x_13; -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_Structure_0__Lean_Elab_Command_expandCtor___spec__16(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +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_14, 0); +x_18 = lean_ctor_get(x_14, 1); +x_19 = lean_unsigned_to_nat(2u); +x_20 = l_Lean_Syntax_getArg(x_1, x_19); +x_21 = l_Lean_Syntax_getArgs(x_20); +lean_dec(x_20); +x_22 = lean_array_get_size(x_21); +x_23 = lean_unsigned_to_nat(0u); +x_24 = lean_nat_dec_lt(x_23, x_22); +if (x_24 == 0) +{ +lean_dec(x_22); +lean_dec(x_21); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_15); lean_dec(x_7); -return x_13; +lean_dec(x_5); +lean_dec(x_3); +lean_ctor_set(x_14, 1, x_13); +lean_ctor_set(x_14, 0, x_2); +return x_14; } 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; uint8_t x_25; lean_object* x_26; uint8_t x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_14 = lean_ctor_get(x_7, 0); -x_15 = lean_ctor_get(x_7, 1); -x_16 = lean_ctor_get(x_7, 2); -x_17 = lean_ctor_get(x_7, 3); -x_18 = lean_ctor_get(x_7, 4); -x_19 = lean_ctor_get(x_7, 5); -x_20 = lean_ctor_get(x_7, 6); -x_21 = lean_ctor_get(x_7, 7); -x_22 = lean_ctor_get(x_7, 8); -x_23 = lean_ctor_get(x_7, 9); -x_24 = lean_ctor_get(x_7, 10); -x_25 = lean_ctor_get_uint8(x_7, sizeof(void*)*12); -x_26 = lean_ctor_get(x_7, 11); -x_27 = lean_ctor_get_uint8(x_7, sizeof(void*)*12 + 1); -lean_inc(x_26); -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_inc(x_15); -lean_inc(x_14); +uint8_t x_25; +x_25 = lean_nat_dec_le(x_22, x_22); +if (x_25 == 0) +{ +lean_dec(x_22); +lean_dec(x_21); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_15); lean_dec(x_7); -x_28 = l_Lean_replaceRef(x_1, x_19); -lean_dec(x_19); -x_29 = lean_alloc_ctor(0, 12, 2); -lean_ctor_set(x_29, 0, x_14); -lean_ctor_set(x_29, 1, x_15); -lean_ctor_set(x_29, 2, x_16); -lean_ctor_set(x_29, 3, x_17); -lean_ctor_set(x_29, 4, x_18); -lean_ctor_set(x_29, 5, x_28); -lean_ctor_set(x_29, 6, x_20); -lean_ctor_set(x_29, 7, x_21); -lean_ctor_set(x_29, 8, x_22); -lean_ctor_set(x_29, 9, x_23); -lean_ctor_set(x_29, 10, x_24); -lean_ctor_set(x_29, 11, x_26); -lean_ctor_set_uint8(x_29, sizeof(void*)*12, x_25); -lean_ctor_set_uint8(x_29, sizeof(void*)*12 + 1, x_27); -x_30 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__16(x_2, x_3, x_4, x_5, x_6, x_29, x_8, x_9); -lean_dec(x_29); -return x_30; +lean_dec(x_5); +lean_dec(x_3); +lean_ctor_set(x_14, 1, x_13); +lean_ctor_set(x_14, 0, x_2); +return x_14; +} +else +{ +size_t x_26; size_t x_27; lean_object* x_28; +lean_free_object(x_14); +x_26 = 0; +x_27 = lean_usize_of_nat(x_22); +lean_dec(x_22); +x_28 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1(x_3, x_4, x_5, x_15, x_17, x_18, x_21, x_26, x_27, x_2, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_21); +return x_28; } } } -static lean_object* _init_l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("unexpected doc string", 21, 21); -return x_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; uint8_t x_36; +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_unsigned_to_nat(2u); +x_32 = l_Lean_Syntax_getArg(x_1, x_31); +x_33 = l_Lean_Syntax_getArgs(x_32); +lean_dec(x_32); +x_34 = lean_array_get_size(x_33); +x_35 = lean_unsigned_to_nat(0u); +x_36 = lean_nat_dec_lt(x_35, x_34); +if (x_36 == 0) +{ +lean_object* x_37; +lean_dec(x_34); +lean_dec(x_33); +lean_dec(x_30); +lean_dec(x_29); +lean_dec(x_15); +lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_3); +x_37 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_37, 0, x_2); +lean_ctor_set(x_37, 1, x_13); +return x_37; } +else +{ +uint8_t x_38; +x_38 = lean_nat_dec_le(x_34, x_34); +if (x_38 == 0) +{ +lean_object* x_39; +lean_dec(x_34); +lean_dec(x_33); +lean_dec(x_30); +lean_dec(x_29); +lean_dec(x_15); +lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_3); +x_39 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_39, 0, x_2); +lean_ctor_set(x_39, 1, x_13); +return x_39; } -static lean_object* _init_l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__2() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +size_t x_40; size_t x_41; lean_object* x_42; +x_40 = 0; +x_41 = lean_usize_of_nat(x_34); +lean_dec(x_34); +x_42 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1(x_3, x_4, x_5, x_15, x_29, x_30, x_33, x_40, x_41, x_2, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_33); +return x_42; } } -static lean_object* _init_l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__3() { +} +} +} +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("", 0, 0); +x_1 = lean_mk_string_unchecked("Parser", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__4() { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__2() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__3; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Term", 4, 4); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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) { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__3() { _start: { -lean_object* x_9; lean_object* x_10; -x_9 = lean_unsigned_to_nat(1u); -x_10 = l_Lean_Syntax_getArg(x_1, x_9); -if (lean_obj_tag(x_10) == 2) -{ -uint8_t x_11; -lean_dec(x_6); -lean_dec(x_2); -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; -x_12 = lean_ctor_get(x_10, 1); -x_13 = lean_ctor_get(x_10, 0); -lean_dec(x_13); -x_14 = lean_string_utf8_byte_size(x_12); -x_15 = lean_unsigned_to_nat(2u); -x_16 = lean_nat_sub(x_14, x_15); -lean_dec(x_14); -x_17 = lean_unsigned_to_nat(0u); -x_18 = lean_string_utf8_extract(x_12, x_17, x_16); -lean_dec(x_16); -lean_dec(x_12); -lean_ctor_set_tag(x_10, 0); -lean_ctor_set(x_10, 1, x_8); -lean_ctor_set(x_10, 0, x_18); -return x_10; -} -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; -x_19 = lean_ctor_get(x_10, 1); -lean_inc(x_19); -lean_dec(x_10); -x_20 = lean_string_utf8_byte_size(x_19); -x_21 = lean_unsigned_to_nat(2u); -x_22 = lean_nat_sub(x_20, x_21); -lean_dec(x_20); -x_23 = lean_unsigned_to_nat(0u); -x_24 = lean_string_utf8_extract(x_19, x_23, x_22); -lean_dec(x_22); -lean_dec(x_19); -x_25 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_25, 0, x_24); -lean_ctor_set(x_25, 1, x_8); -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_object* x_31; lean_object* x_32; -x_26 = l_Lean_MessageData_ofSyntax(x_10); -x_27 = l_Lean_indentD(x_26); -x_28 = l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__2; -x_29 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_29, 0, x_28); -lean_ctor_set(x_29, 1, x_27); -x_30 = l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__4; -x_31 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_31, 0, x_29); -lean_ctor_set(x_31, 1, x_30); -x_32 = l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__15(x_1, x_31, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -return x_32; -} +lean_object* x_1; +x_1 = lean_mk_string_unchecked("binderTactic", 12, 12); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, uint8_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__4() { _start: { -uint8_t x_14; uint8_t x_15; -x_14 = l_Lean_Syntax_isNone(x_1); -x_15 = l_Lean_Syntax_isNone(x_2); -if (x_14 == 0) -{ -if (x_15 == 0) -{ -uint8_t x_16; lean_object* x_17; lean_object* x_18; -x_16 = 1; -x_17 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_17, 0, x_3); -lean_ctor_set(x_17, 1, x_6); -lean_ctor_set_uint8(x_17, sizeof(void*)*2, x_4); -lean_ctor_set_uint8(x_17, sizeof(void*)*2 + 1, x_16); -lean_ctor_set_uint8(x_17, sizeof(void*)*2 + 2, x_5); -lean_ctor_set_uint8(x_17, sizeof(void*)*2 + 3, x_16); -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_17); -lean_ctor_set(x_18, 1, x_13); -return x_18; -} -else -{ -uint8_t x_19; uint8_t x_20; lean_object* x_21; lean_object* x_22; -x_19 = 1; -x_20 = 0; -x_21 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_21, 0, x_3); -lean_ctor_set(x_21, 1, x_6); -lean_ctor_set_uint8(x_21, sizeof(void*)*2, x_4); -lean_ctor_set_uint8(x_21, sizeof(void*)*2 + 1, x_19); -lean_ctor_set_uint8(x_21, sizeof(void*)*2 + 2, x_5); -lean_ctor_set_uint8(x_21, sizeof(void*)*2 + 3, x_20); -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_21); -lean_ctor_set(x_22, 1, x_13); -return x_22; -} +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__6; +x_2 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__1; +x_3 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__2; +x_4 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__3; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; } -else -{ -if (x_15 == 0) -{ -uint8_t x_23; uint8_t x_24; lean_object* x_25; lean_object* x_26; -x_23 = 0; -x_24 = 1; -x_25 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_25, 0, x_3); -lean_ctor_set(x_25, 1, x_6); -lean_ctor_set_uint8(x_25, sizeof(void*)*2, x_4); -lean_ctor_set_uint8(x_25, sizeof(void*)*2 + 1, x_23); -lean_ctor_set_uint8(x_25, sizeof(void*)*2 + 2, x_5); -lean_ctor_set_uint8(x_25, sizeof(void*)*2 + 3, x_24); -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_26, 1, x_13); -return x_26; } -else +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__5() { +_start: { -uint8_t x_27; lean_object* x_28; lean_object* x_29; -x_27 = 0; -x_28 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_28, 0, x_3); -lean_ctor_set(x_28, 1, x_6); -lean_ctor_set_uint8(x_28, sizeof(void*)*2, x_4); -lean_ctor_set_uint8(x_28, sizeof(void*)*2 + 1, x_27); -lean_ctor_set_uint8(x_28, sizeof(void*)*2 + 2, x_5); -lean_ctor_set_uint8(x_28, sizeof(void*)*2 + 3, x_27); -x_29 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_29, 0, x_28); -lean_ctor_set(x_29, 1, x_13); -return x_29; -} -} +lean_object* x_1; +x_1 = lean_mk_string_unchecked("invalid field declaration, type must be provided when auto-param (tactic) is used", 81, 81); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__6() { _start: { -lean_object* x_14; -x_14 = l_Lean_Syntax_getOptional_x3f(x_5); -if (lean_obj_tag(x_14) == 0) -{ -lean_object* x_15; lean_object* x_16; -x_15 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; -x_16 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__1(x_1, x_2, x_3, x_6, x_4, x_15, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_11); -lean_dec(x_7); -return x_16; -} -else -{ -lean_object* x_17; lean_object* x_18; -x_17 = lean_ctor_get(x_14, 0); -lean_inc(x_17); -lean_dec(x_14); -lean_inc(x_11); -lean_inc(x_7); -x_18 = l_Lean_Elab_elabDeclAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__2(x_17, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_17); -if (lean_obj_tag(x_18) == 0) -{ -lean_object* x_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_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__1(x_1, x_2, x_3, x_6, x_4, x_19, x_7, x_8, x_9, x_10, x_11, x_12, x_20); -lean_dec(x_11); -lean_dec(x_7); -return x_21; +lean_object* x_1; lean_object* x_2; +x_1 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__5; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } -else -{ -uint8_t x_22; -lean_dec(x_11); -lean_dec(x_7); -lean_dec(x_3); -x_22 = !lean_is_exclusive(x_18); -if (x_22 == 0) -{ -return x_18; } -else +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__7() { +_start: { -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_1; +x_1 = lean_mk_string_unchecked("forall", 6, 6); +return x_1; } } -static lean_object* _init_l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__1() { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__8() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Command", 7, 7); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__6; +x_2 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__1; +x_3 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__2; +x_4 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__7; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; } } -static lean_object* _init_l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__2() { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__9() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("private", 7, 7); +x_1 = lean_mk_string_unchecked("null", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__3() { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__10() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__1; -x_2 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__2; -x_3 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__1; -x_4 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__2; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__9; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -static lean_object* _init_l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__4() { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__11() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("protected", 9, 9); +x_1 = lean_mk_string_unchecked("app", 3, 3); return x_1; } } -static lean_object* _init_l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__5() { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__1; -x_2 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__2; -x_3 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__1; -x_4 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__4; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__6; +x_2 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__1; +x_3 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__2; +x_4 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__11; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__6() { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__13() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("unexpected visibility modifier", 30, 30); +x_1 = lean_mk_string_unchecked("autoParam", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__7() { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__14() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__6; -x_2 = l_Lean_stringToMessageData(x_1); +x_1 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__13; +x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__15() { _start: { -lean_object* x_14; -x_14 = l_Lean_Syntax_getOptional_x3f(x_5); -if (lean_obj_tag(x_14) == 0) -{ -uint8_t x_15; lean_object* x_16; -x_15 = 0; -x_16 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__2(x_1, x_2, x_6, x_3, x_4, x_15, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -return x_16; -} -else -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; -x_17 = lean_ctor_get(x_14, 0); -lean_inc(x_17); -lean_dec(x_14); -lean_inc(x_17); -x_18 = l_Lean_Syntax_getKind(x_17); -x_19 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__3; -x_20 = lean_name_eq(x_18, x_19); -if (x_20 == 0) -{ -lean_object* x_21; uint8_t x_22; -x_21 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__5; -x_22 = lean_name_eq(x_18, x_21); -lean_dec(x_18); -if (x_22 == 0) -{ -lean_object* x_23; lean_object* x_24; uint8_t x_25; -lean_dec(x_6); -x_23 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__7; -x_24 = l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__12(x_17, x_23, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_17); -x_25 = !lean_is_exclusive(x_24); -if (x_25 == 0) -{ -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(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_object* x_30; -lean_dec(x_17); -x_29 = 1; -x_30 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__2(x_1, x_2, x_6, x_3, x_4, x_29, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -return x_30; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__13; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -else +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__16() { +_start: { -uint8_t x_31; lean_object* x_32; -lean_dec(x_18); -lean_dec(x_17); -x_31 = 2; -x_32 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__2(x_1, x_2, x_6, x_3, x_4, x_31, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -return x_32; -} -} +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__15; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; } } -static lean_object* _init_l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___closed__1() { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__17() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("partial", 7, 7); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__16; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; } } -static lean_object* _init_l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___closed__2() { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__18() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__1; -x_2 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__2; -x_3 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__1; -x_4 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___closed__1; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = lean_box(2); +x_2 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__10; +x_3 = l_Lean_Elab_Command_instInhabitedStructCtorView___closed__1; +x_4 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _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; uint8_t x_21; lean_object* x_22; uint8_t x_23; -x_9 = lean_unsigned_to_nat(0u); -x_10 = l_Lean_Syntax_getArg(x_1, x_9); -x_11 = lean_unsigned_to_nat(1u); -x_12 = l_Lean_Syntax_getArg(x_1, x_11); -x_13 = lean_unsigned_to_nat(2u); -x_14 = l_Lean_Syntax_getArg(x_1, x_13); -x_15 = lean_unsigned_to_nat(3u); -x_16 = l_Lean_Syntax_getArg(x_1, x_15); -x_17 = lean_unsigned_to_nat(4u); -x_18 = l_Lean_Syntax_getArg(x_1, x_17); -x_19 = lean_unsigned_to_nat(5u); -x_20 = l_Lean_Syntax_getArg(x_1, x_19); -x_21 = l_Lean_Syntax_isNone(x_20); -x_22 = l_Lean_Syntax_getOptional_x3f(x_10); -lean_dec(x_10); -if (x_21 == 0) +uint8_t x_14; uint8_t x_15; +x_14 = 0; +x_15 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_404_(x_4, x_14); +if (x_15 == 0) { -lean_object* x_47; lean_object* x_48; lean_object* x_49; uint8_t x_50; -x_47 = l_Lean_Syntax_getArg(x_20, x_9); -lean_dec(x_20); -x_48 = l_Lean_Syntax_getKind(x_47); -x_49 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___closed__2; -x_50 = lean_name_eq(x_48, x_49); -lean_dec(x_48); -if (x_50 == 0) +lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; +x_16 = lean_unsigned_to_nat(3u); +x_17 = l_Lean_Syntax_getArg(x_1, x_16); +x_18 = l_Lean_Elab_expandDeclSig(x_17); +lean_dec(x_17); +x_19 = !lean_is_exclusive(x_18); +if (x_19 == 0) { -uint8_t x_51; -x_51 = 1; -x_23 = x_51; -goto block_46; +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_20 = lean_ctor_get(x_18, 0); +x_21 = lean_ctor_get(x_18, 1); +x_22 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_22, 0, x_21); +x_23 = lean_box(0); +lean_ctor_set(x_18, 1, x_23); +lean_ctor_set(x_18, 0, x_22); +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_20); +lean_ctor_set(x_24, 1, x_18); +x_25 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__1(x_1, x_2, x_3, x_4, x_5, x_24, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +return x_25; } else { -uint8_t x_52; -x_52 = 0; -x_23 = x_52; -goto block_46; +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_26 = lean_ctor_get(x_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, 1, 0); +lean_ctor_set(x_28, 0, x_27); +x_29 = lean_box(0); +x_30 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_26); +lean_ctor_set(x_31, 1, x_30); +x_32 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__1(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); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +return x_32; } } else { -uint8_t x_53; -lean_dec(x_20); -x_53 = 2; -x_23 = x_53; -goto block_46; -} -block_46: -{ -if (lean_obj_tag(x_22) == 0) -{ -lean_object* x_24; lean_object* x_25; -x_24 = lean_box(0); -x_25 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3(x_16, x_18, x_23, x_12, x_14, x_24, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_14); -lean_dec(x_12); -lean_dec(x_18); -lean_dec(x_16); -return x_25; -} -else +lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; +x_33 = lean_unsigned_to_nat(3u); +x_34 = l_Lean_Syntax_getArg(x_1, x_33); +x_35 = l_Lean_Elab_expandOptDeclSig(x_34); +lean_dec(x_34); +x_36 = !lean_is_exclusive(x_35); +if (x_36 == 0) { -uint8_t x_26; -x_26 = !lean_is_exclusive(x_22); -if (x_26 == 0) +lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; +x_37 = lean_ctor_get(x_35, 0); +x_38 = lean_ctor_get(x_35, 1); +x_39 = lean_unsigned_to_nat(4u); +x_40 = l_Lean_Syntax_getArg(x_1, x_39); +x_41 = l_Lean_Syntax_isNone(x_40); +if (x_41 == 0) { -lean_object* x_27; lean_object* x_28; -x_27 = lean_ctor_get(x_22, 0); -lean_inc(x_6); -lean_inc(x_2); -x_28 = l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14(x_27, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_27); -if (lean_obj_tag(x_28) == 0) +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; uint8_t x_46; +x_42 = lean_unsigned_to_nat(0u); +x_43 = l_Lean_Syntax_getArg(x_40, x_42); +lean_dec(x_40); +lean_inc(x_43); +x_44 = l_Lean_Syntax_getKind(x_43); +x_45 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__4; +x_46 = lean_name_eq(x_44, x_45); +lean_dec(x_44); +if (x_46 == 0) { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_28, 0); -lean_inc(x_29); -x_30 = lean_ctor_get(x_28, 1); -lean_inc(x_30); -lean_dec(x_28); -lean_ctor_set(x_22, 0, x_29); -x_31 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3(x_16, x_18, x_23, x_12, x_14, x_22, x_2, x_3, x_4, x_5, x_6, x_7, x_30); -lean_dec(x_14); +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_47 = lean_unsigned_to_nat(1u); +x_48 = l_Lean_Syntax_getArg(x_43, x_47); +lean_dec(x_43); +x_49 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_49, 0, x_48); +lean_ctor_set(x_35, 1, x_49); +lean_ctor_set(x_35, 0, x_38); +x_50 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_50, 0, x_37); +lean_ctor_set(x_50, 1, x_35); +x_51 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__1(x_1, x_2, x_3, x_4, x_5, x_50, x_7, x_8, x_9, x_10, x_11, x_12, x_13); lean_dec(x_12); -lean_dec(x_18); -lean_dec(x_16); -return x_31; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +return x_51; } else { -uint8_t x_32; -lean_free_object(x_22); -lean_dec(x_18); -lean_dec(x_16); -lean_dec(x_14); -lean_dec(x_12); -lean_dec(x_6); +if (lean_obj_tag(x_38) == 0) +{ +lean_object* x_52; lean_object* x_53; uint8_t x_54; +lean_free_object(x_35); +lean_dec(x_37); +lean_dec(x_5); +lean_dec(x_3); lean_dec(x_2); -x_32 = !lean_is_exclusive(x_28); -if (x_32 == 0) +x_52 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__6; +x_53 = l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__2(x_43, x_52, 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_43); +x_54 = !lean_is_exclusive(x_53); +if (x_54 == 0) { -return x_28; +return x_53; } else { -lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_33 = lean_ctor_get(x_28, 0); -x_34 = lean_ctor_get(x_28, 1); -lean_inc(x_34); -lean_inc(x_33); -lean_dec(x_28); -x_35 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_35, 0, x_33); -lean_ctor_set(x_35, 1, x_34); -return x_35; -} +lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_55 = lean_ctor_get(x_53, 0); +x_56 = lean_ctor_get(x_53, 1); +lean_inc(x_56); +lean_inc(x_55); +lean_dec(x_53); +x_57 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_57, 0, x_55); +lean_ctor_set(x_57, 1, x_56); +return x_57; } } else { -lean_object* x_36; lean_object* x_37; -x_36 = lean_ctor_get(x_22, 0); -lean_inc(x_36); -lean_dec(x_22); -lean_inc(x_6); -lean_inc(x_2); -x_37 = l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14(x_36, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_36); -if (lean_obj_tag(x_37) == 0) +uint8_t x_58; +x_58 = !lean_is_exclusive(x_38); +if (x_58 == 0) { -lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_38 = lean_ctor_get(x_37, 0); -lean_inc(x_38); -x_39 = lean_ctor_get(x_37, 1); -lean_inc(x_39); +lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; +x_59 = lean_ctor_get(x_38, 0); +x_60 = lean_unsigned_to_nat(2u); +x_61 = l_Lean_Syntax_getArg(x_43, x_60); +lean_dec(x_43); +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_61); +x_62 = l_Lean_Elab_Term_declareTacticSyntax(x_61, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_62) == 0) +{ +lean_object* x_63; lean_object* x_64; lean_object* x_65; uint8_t x_66; lean_object* x_67; lean_object* x_68; uint8_t x_69; +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_11, 5); +lean_inc(x_65); +x_66 = 0; +x_67 = l_Lean_SourceInfo_fromRef(x_65, x_66); +lean_dec(x_65); +x_68 = lean_st_ref_get(x_12, x_64); +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; uint8_t x_85; +x_70 = lean_ctor_get(x_68, 1); +x_71 = lean_ctor_get(x_68, 0); +lean_dec(x_71); +x_72 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__7; +lean_inc(x_67); +lean_ctor_set_tag(x_68, 2); +lean_ctor_set(x_68, 1, x_72); +lean_ctor_set(x_68, 0, x_67); +x_73 = l_Lean_Syntax_getArgs(x_37); lean_dec(x_37); -x_40 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_40, 0, x_38); -x_41 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3(x_16, x_18, x_23, x_12, x_14, x_40, x_2, x_3, x_4, x_5, x_6, x_7, x_39); -lean_dec(x_14); +x_74 = l_Lean_Elab_Command_instInhabitedStructCtorView___closed__1; +x_75 = l_Array_append___rarg(x_74, x_73); +lean_dec(x_73); +x_76 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__10; +lean_inc(x_67); +x_77 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_77, 0, x_67); +lean_ctor_set(x_77, 1, x_76); +lean_ctor_set(x_77, 2, x_75); +lean_inc(x_67); +x_78 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_78, 0, x_67); +lean_ctor_set(x_78, 1, x_76); +lean_ctor_set(x_78, 2, x_74); +x_79 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__8; +lean_inc(x_67); +x_80 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_80, 0, x_67); +lean_ctor_set(x_80, 1, x_79); +x_81 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__8; +lean_inc(x_67); +x_82 = l_Lean_Syntax_node5(x_67, x_81, x_68, x_77, x_78, x_80, x_59); +x_83 = lean_ctor_get(x_11, 10); +lean_inc(x_83); +x_84 = lean_st_ref_get(x_12, x_70); +x_85 = !lean_is_exclusive(x_84); +if (x_85 == 0) +{ +lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; +x_86 = lean_ctor_get(x_84, 0); +x_87 = lean_ctor_get(x_84, 1); +x_88 = lean_ctor_get(x_86, 0); +lean_inc(x_88); +lean_dec(x_86); +x_89 = lean_environment_main_module(x_88); +x_90 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__15; +x_91 = l_Lean_addMacroScope(x_89, x_90, x_83); +x_92 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__14; +x_93 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__17; +lean_inc(x_67); +x_94 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_94, 0, x_67); +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_mkIdentFrom(x_61, x_63, x_66); +lean_dec(x_61); +lean_inc(x_67); +x_96 = l_Lean_Syntax_node2(x_67, x_76, x_82, x_95); +x_97 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__12; +x_98 = l_Lean_Syntax_node2(x_67, x_97, x_94, x_96); +lean_ctor_set(x_38, 0, x_98); +x_99 = lean_box(0); +lean_ctor_set(x_35, 1, x_99); +lean_ctor_set(x_35, 0, x_38); +x_100 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__18; +lean_ctor_set(x_84, 1, x_35); +lean_ctor_set(x_84, 0, x_100); +x_101 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__1(x_1, x_2, x_3, x_4, x_5, x_84, x_7, x_8, x_9, x_10, x_11, x_12, x_87); lean_dec(x_12); -lean_dec(x_18); -lean_dec(x_16); -return x_41; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +return x_101; } else { -lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; -lean_dec(x_18); -lean_dec(x_16); -lean_dec(x_14); +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; +x_102 = lean_ctor_get(x_84, 0); +x_103 = lean_ctor_get(x_84, 1); +lean_inc(x_103); +lean_inc(x_102); +lean_dec(x_84); +x_104 = lean_ctor_get(x_102, 0); +lean_inc(x_104); +lean_dec(x_102); +x_105 = lean_environment_main_module(x_104); +x_106 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__15; +x_107 = l_Lean_addMacroScope(x_105, x_106, x_83); +x_108 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__14; +x_109 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__17; +lean_inc(x_67); +x_110 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_110, 0, x_67); +lean_ctor_set(x_110, 1, x_108); +lean_ctor_set(x_110, 2, x_107); +lean_ctor_set(x_110, 3, x_109); +x_111 = l_Lean_mkIdentFrom(x_61, x_63, x_66); +lean_dec(x_61); +lean_inc(x_67); +x_112 = l_Lean_Syntax_node2(x_67, x_76, x_82, x_111); +x_113 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__12; +x_114 = l_Lean_Syntax_node2(x_67, x_113, x_110, x_112); +lean_ctor_set(x_38, 0, x_114); +x_115 = lean_box(0); +lean_ctor_set(x_35, 1, x_115); +lean_ctor_set(x_35, 0, x_38); +x_116 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__18; +x_117 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_117, 0, x_116); +lean_ctor_set(x_117, 1, x_35); +x_118 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__1(x_1, x_2, x_3, x_4, x_5, x_117, x_7, x_8, x_9, x_10, x_11, x_12, x_103); lean_dec(x_12); -lean_dec(x_6); -lean_dec(x_2); -x_42 = lean_ctor_get(x_37, 0); -lean_inc(x_42); -x_43 = lean_ctor_get(x_37, 1); -lean_inc(x_43); -if (lean_is_exclusive(x_37)) { - lean_ctor_release(x_37, 0); - lean_ctor_release(x_37, 1); - x_44 = x_37; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +return x_118; +} +} +else +{ +lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; +x_119 = lean_ctor_get(x_68, 1); +lean_inc(x_119); +lean_dec(x_68); +x_120 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__7; +lean_inc(x_67); +x_121 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_121, 0, x_67); +lean_ctor_set(x_121, 1, x_120); +x_122 = l_Lean_Syntax_getArgs(x_37); +lean_dec(x_37); +x_123 = l_Lean_Elab_Command_instInhabitedStructCtorView___closed__1; +x_124 = l_Array_append___rarg(x_123, x_122); +lean_dec(x_122); +x_125 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__10; +lean_inc(x_67); +x_126 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_126, 0, x_67); +lean_ctor_set(x_126, 1, x_125); +lean_ctor_set(x_126, 2, x_124); +lean_inc(x_67); +x_127 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_127, 0, x_67); +lean_ctor_set(x_127, 1, x_125); +lean_ctor_set(x_127, 2, x_123); +x_128 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__8; +lean_inc(x_67); +x_129 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_129, 0, x_67); +lean_ctor_set(x_129, 1, x_128); +x_130 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__8; +lean_inc(x_67); +x_131 = l_Lean_Syntax_node5(x_67, x_130, x_121, x_126, x_127, x_129, x_59); +x_132 = lean_ctor_get(x_11, 10); +lean_inc(x_132); +x_133 = lean_st_ref_get(x_12, x_119); +x_134 = lean_ctor_get(x_133, 0); +lean_inc(x_134); +x_135 = lean_ctor_get(x_133, 1); +lean_inc(x_135); +if (lean_is_exclusive(x_133)) { + lean_ctor_release(x_133, 0); + lean_ctor_release(x_133, 1); + x_136 = x_133; } else { - lean_dec_ref(x_37); - x_44 = lean_box(0); + lean_dec_ref(x_133); + x_136 = lean_box(0); } -if (lean_is_scalar(x_44)) { - x_45 = lean_alloc_ctor(1, 2, 0); +x_137 = lean_ctor_get(x_134, 0); +lean_inc(x_137); +lean_dec(x_134); +x_138 = lean_environment_main_module(x_137); +x_139 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__15; +x_140 = l_Lean_addMacroScope(x_138, x_139, x_132); +x_141 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__14; +x_142 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__17; +lean_inc(x_67); +x_143 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_143, 0, x_67); +lean_ctor_set(x_143, 1, x_141); +lean_ctor_set(x_143, 2, x_140); +lean_ctor_set(x_143, 3, x_142); +x_144 = l_Lean_mkIdentFrom(x_61, x_63, x_66); +lean_dec(x_61); +lean_inc(x_67); +x_145 = l_Lean_Syntax_node2(x_67, x_125, x_131, x_144); +x_146 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__12; +x_147 = l_Lean_Syntax_node2(x_67, x_146, x_143, x_145); +lean_ctor_set(x_38, 0, x_147); +x_148 = lean_box(0); +lean_ctor_set(x_35, 1, x_148); +lean_ctor_set(x_35, 0, x_38); +x_149 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__18; +if (lean_is_scalar(x_136)) { + x_150 = lean_alloc_ctor(0, 2, 0); } else { - x_45 = x_44; + x_150 = x_136; } -lean_ctor_set(x_45, 0, x_42); -lean_ctor_set(x_45, 1, x_43); -return x_45; +lean_ctor_set(x_150, 0, x_149); +lean_ctor_set(x_150, 1, x_35); +x_151 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__1(x_1, x_2, x_3, x_4, x_5, x_150, x_7, x_8, x_9, x_10, x_11, x_12, x_135); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +return x_151; } } +else +{ +uint8_t x_152; +lean_dec(x_61); +lean_free_object(x_38); +lean_dec(x_59); +lean_free_object(x_35); +lean_dec(x_37); +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_3); +lean_dec(x_2); +x_152 = !lean_is_exclusive(x_62); +if (x_152 == 0) +{ +return x_62; } +else +{ +lean_object* x_153; lean_object* x_154; lean_object* x_155; +x_153 = lean_ctor_get(x_62, 0); +x_154 = lean_ctor_get(x_62, 1); +lean_inc(x_154); +lean_inc(x_153); +lean_dec(x_62); +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; } } } -static lean_object* _init_l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__1___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("invalid use of attributes in constructor declaration", 52, 52); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__1___closed__2() { -_start: +lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; +x_156 = lean_ctor_get(x_38, 0); +lean_inc(x_156); +lean_dec(x_38); +x_157 = lean_unsigned_to_nat(2u); +x_158 = l_Lean_Syntax_getArg(x_43, x_157); +lean_dec(x_43); +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_158); +x_159 = l_Lean_Elab_Term_declareTacticSyntax(x_158, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_159) == 0) { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__1___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +lean_object* x_160; lean_object* x_161; lean_object* x_162; uint8_t x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; 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_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_11, 5); +lean_inc(x_162); +x_163 = 0; +x_164 = l_Lean_SourceInfo_fromRef(x_162, x_163); +lean_dec(x_162); +x_165 = lean_st_ref_get(x_12, x_161); +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; +} else { + lean_dec_ref(x_165); + x_167 = lean_box(0); } +x_168 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__7; +lean_inc(x_164); +if (lean_is_scalar(x_167)) { + x_169 = lean_alloc_ctor(2, 2, 0); +} else { + x_169 = x_167; + lean_ctor_set_tag(x_169, 2); } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_10 = lean_ctor_get(x_1, 1); -x_11 = lean_array_get_size(x_10); -x_12 = lean_unsigned_to_nat(0u); -x_13 = lean_nat_dec_eq(x_11, x_12); +lean_ctor_set(x_169, 0, x_164); +lean_ctor_set(x_169, 1, x_168); +x_170 = l_Lean_Syntax_getArgs(x_37); +lean_dec(x_37); +x_171 = l_Lean_Elab_Command_instInhabitedStructCtorView___closed__1; +x_172 = l_Array_append___rarg(x_171, x_170); +lean_dec(x_170); +x_173 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__10; +lean_inc(x_164); +x_174 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_174, 0, x_164); +lean_ctor_set(x_174, 1, x_173); +lean_ctor_set(x_174, 2, x_172); +lean_inc(x_164); +x_175 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_175, 0, x_164); +lean_ctor_set(x_175, 1, x_173); +lean_ctor_set(x_175, 2, x_171); +x_176 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__8; +lean_inc(x_164); +x_177 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_177, 0, x_164); +lean_ctor_set(x_177, 1, x_176); +x_178 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__8; +lean_inc(x_164); +x_179 = l_Lean_Syntax_node5(x_164, x_178, x_169, x_174, x_175, x_177, x_156); +x_180 = lean_ctor_get(x_11, 10); +lean_inc(x_180); +x_181 = lean_st_ref_get(x_12, x_166); +x_182 = lean_ctor_get(x_181, 0); +lean_inc(x_182); +x_183 = lean_ctor_get(x_181, 1); +lean_inc(x_183); +if (lean_is_exclusive(x_181)) { + lean_ctor_release(x_181, 0); + lean_ctor_release(x_181, 1); + x_184 = x_181; +} else { + lean_dec_ref(x_181); + x_184 = lean_box(0); +} +x_185 = lean_ctor_get(x_182, 0); +lean_inc(x_185); +lean_dec(x_182); +x_186 = lean_environment_main_module(x_185); +x_187 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__15; +x_188 = l_Lean_addMacroScope(x_186, x_187, x_180); +x_189 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__14; +x_190 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__17; +lean_inc(x_164); +x_191 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_191, 0, x_164); +lean_ctor_set(x_191, 1, x_189); +lean_ctor_set(x_191, 2, x_188); +lean_ctor_set(x_191, 3, x_190); +x_192 = l_Lean_mkIdentFrom(x_158, x_160, x_163); +lean_dec(x_158); +lean_inc(x_164); +x_193 = l_Lean_Syntax_node2(x_164, x_173, x_179, x_192); +x_194 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__12; +x_195 = l_Lean_Syntax_node2(x_164, x_194, x_191, x_193); +x_196 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_196, 0, x_195); +x_197 = lean_box(0); +lean_ctor_set(x_35, 1, x_197); +lean_ctor_set(x_35, 0, x_196); +x_198 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__18; +if (lean_is_scalar(x_184)) { + x_199 = lean_alloc_ctor(0, 2, 0); +} else { + x_199 = x_184; +} +lean_ctor_set(x_199, 0, x_198); +lean_ctor_set(x_199, 1, x_35); +x_200 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__1(x_1, x_2, x_3, x_4, x_5, x_199, x_7, x_8, x_9, x_10, x_11, x_12, x_183); +lean_dec(x_12); lean_dec(x_11); -if (x_13 == 0) -{ -lean_object* x_14; lean_object* x_15; -x_14 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__1___closed__2; -x_15 = l_Lean_throwError___at_Lean_Elab_Term_throwErrorIfErrors___spec__1(x_14, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_15; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +return x_200; } else { -lean_object* x_16; lean_object* x_17; +lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; +lean_dec(x_158); +lean_dec(x_156); +lean_free_object(x_35); +lean_dec(x_37); +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_3); -x_16 = lean_box(0); -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_16); -lean_ctor_set(x_17, 1, x_9); -return x_17; +lean_dec(x_2); +x_201 = lean_ctor_get(x_159, 0); +lean_inc(x_201); +x_202 = lean_ctor_get(x_159, 1); +lean_inc(x_202); +if (lean_is_exclusive(x_159)) { + lean_ctor_release(x_159, 0); + lean_ctor_release(x_159, 1); + x_203 = x_159; +} else { + lean_dec_ref(x_159); + x_203 = lean_box(0); } +if (lean_is_scalar(x_203)) { + x_204 = lean_alloc_ctor(1, 2, 0); +} else { + x_204 = x_203; } +lean_ctor_set(x_204, 0, x_201); +lean_ctor_set(x_204, 1, x_202); +return x_204; } -static lean_object* _init_l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__2___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("invalid use of 'unsafe' in constructor declaration", 50, 50); -return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__2___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__2___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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) { -_start: -{ -uint8_t x_10; -x_10 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 3); -if (x_10 == 0) +else { -lean_object* x_11; lean_object* x_12; -x_11 = lean_box(0); -x_12 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__1(x_1, x_11, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_12; +lean_object* x_205; lean_object* x_206; lean_object* x_207; +lean_dec(x_40); +x_205 = lean_box(0); +lean_ctor_set(x_35, 1, x_205); +lean_ctor_set(x_35, 0, x_38); +x_206 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_206, 0, x_37); +lean_ctor_set(x_206, 1, x_35); +x_207 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__1(x_1, x_2, x_3, x_4, x_5, x_206, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +return x_207; +} } else { -lean_object* x_13; lean_object* x_14; uint8_t x_15; -x_13 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__2___closed__2; -x_14 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -x_15 = !lean_is_exclusive(x_14); -if (x_15 == 0) +lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; uint8_t x_212; +x_208 = lean_ctor_get(x_35, 0); +x_209 = lean_ctor_get(x_35, 1); +lean_inc(x_209); +lean_inc(x_208); +lean_dec(x_35); +x_210 = lean_unsigned_to_nat(4u); +x_211 = l_Lean_Syntax_getArg(x_1, x_210); +x_212 = l_Lean_Syntax_isNone(x_211); +if (x_212 == 0) { -return x_14; +lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; uint8_t x_217; +x_213 = lean_unsigned_to_nat(0u); +x_214 = l_Lean_Syntax_getArg(x_211, x_213); +lean_dec(x_211); +lean_inc(x_214); +x_215 = l_Lean_Syntax_getKind(x_214); +x_216 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__4; +x_217 = lean_name_eq(x_215, x_216); +lean_dec(x_215); +if (x_217 == 0) +{ +lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; +x_218 = lean_unsigned_to_nat(1u); +x_219 = l_Lean_Syntax_getArg(x_214, x_218); +lean_dec(x_214); +x_220 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_220, 0, x_219); +x_221 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_221, 0, x_209); +lean_ctor_set(x_221, 1, x_220); +x_222 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_222, 0, x_208); +lean_ctor_set(x_222, 1, x_221); +x_223 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__1(x_1, x_2, x_3, x_4, x_5, x_222, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +return x_223; } else { -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_14, 0); -x_17 = lean_ctor_get(x_14, 1); -lean_inc(x_17); -lean_inc(x_16); -lean_dec(x_14); -x_18 = lean_alloc_ctor(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_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__3___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("invalid use of 'partial' in constructor declaration", 51, 51); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__3___closed__2() { -_start: +if (lean_obj_tag(x_209) == 0) { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__3___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +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_dec(x_208); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +x_224 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__6; +x_225 = l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__2(x_214, x_224, 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_214); +x_226 = lean_ctor_get(x_225, 0); +lean_inc(x_226); +x_227 = lean_ctor_get(x_225, 1); +lean_inc(x_227); +if (lean_is_exclusive(x_225)) { + lean_ctor_release(x_225, 0); + lean_ctor_release(x_225, 1); + x_228 = x_225; +} else { + lean_dec_ref(x_225); + x_228 = lean_box(0); } +if (lean_is_scalar(x_228)) { + x_229 = lean_alloc_ctor(1, 2, 0); +} else { + x_229 = x_228; } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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) { -_start: -{ -uint8_t x_10; -x_10 = l_Lean_Elab_Modifiers_isPartial(x_1); -if (x_10 == 0) -{ -lean_object* x_11; lean_object* x_12; -x_11 = lean_box(0); -x_12 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__2(x_1, x_11, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_12; +lean_ctor_set(x_229, 0, x_226); +lean_ctor_set(x_229, 1, x_227); +return x_229; } else { -lean_object* x_13; lean_object* x_14; uint8_t x_15; -x_13 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__3___closed__2; -x_14 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -x_15 = !lean_is_exclusive(x_14); -if (x_15 == 0) -{ -return x_14; +lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; +x_230 = lean_ctor_get(x_209, 0); +lean_inc(x_230); +if (lean_is_exclusive(x_209)) { + lean_ctor_release(x_209, 0); + x_231 = x_209; +} else { + lean_dec_ref(x_209); + x_231 = lean_box(0); } -else +x_232 = lean_unsigned_to_nat(2u); +x_233 = l_Lean_Syntax_getArg(x_214, x_232); +lean_dec(x_214); +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_233); +x_234 = l_Lean_Elab_Term_declareTacticSyntax(x_233, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_234) == 0) { -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_14, 0); -x_17 = lean_ctor_get(x_14, 1); -lean_inc(x_17); -lean_inc(x_16); -lean_dec(x_14); -x_18 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_18, 0, x_16); -lean_ctor_set(x_18, 1, x_17); -return x_18; +lean_object* x_235; lean_object* x_236; lean_object* x_237; uint8_t 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_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_ctor_get(x_11, 5); +lean_inc(x_237); +x_238 = 0; +x_239 = l_Lean_SourceInfo_fromRef(x_237, x_238); +lean_dec(x_237); +x_240 = lean_st_ref_get(x_12, x_236); +x_241 = lean_ctor_get(x_240, 1); +lean_inc(x_241); +if (lean_is_exclusive(x_240)) { + lean_ctor_release(x_240, 0); + lean_ctor_release(x_240, 1); + x_242 = x_240; +} else { + lean_dec_ref(x_240); + x_242 = lean_box(0); } +x_243 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__7; +lean_inc(x_239); +if (lean_is_scalar(x_242)) { + x_244 = lean_alloc_ctor(2, 2, 0); +} else { + x_244 = x_242; + lean_ctor_set_tag(x_244, 2); } +lean_ctor_set(x_244, 0, x_239); +lean_ctor_set(x_244, 1, x_243); +x_245 = l_Lean_Syntax_getArgs(x_208); +lean_dec(x_208); +x_246 = l_Lean_Elab_Command_instInhabitedStructCtorView___closed__1; +x_247 = l_Array_append___rarg(x_246, x_245); +lean_dec(x_245); +x_248 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__10; +lean_inc(x_239); +x_249 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_249, 0, x_239); +lean_ctor_set(x_249, 1, x_248); +lean_ctor_set(x_249, 2, x_247); +lean_inc(x_239); +x_250 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_250, 0, x_239); +lean_ctor_set(x_250, 1, x_248); +lean_ctor_set(x_250, 2, x_246); +x_251 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__8; +lean_inc(x_239); +x_252 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_252, 0, x_239); +lean_ctor_set(x_252, 1, x_251); +x_253 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__8; +lean_inc(x_239); +x_254 = l_Lean_Syntax_node5(x_239, x_253, x_244, x_249, x_250, x_252, x_230); +x_255 = lean_ctor_get(x_11, 10); +lean_inc(x_255); +x_256 = lean_st_ref_get(x_12, x_241); +x_257 = lean_ctor_get(x_256, 0); +lean_inc(x_257); +x_258 = lean_ctor_get(x_256, 1); +lean_inc(x_258); +if (lean_is_exclusive(x_256)) { + lean_ctor_release(x_256, 0); + lean_ctor_release(x_256, 1); + x_259 = x_256; +} else { + lean_dec_ref(x_256); + x_259 = lean_box(0); } +x_260 = lean_ctor_get(x_257, 0); +lean_inc(x_260); +lean_dec(x_257); +x_261 = lean_environment_main_module(x_260); +x_262 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__15; +x_263 = l_Lean_addMacroScope(x_261, x_262, x_255); +x_264 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__14; +x_265 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__17; +lean_inc(x_239); +x_266 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_266, 0, x_239); +lean_ctor_set(x_266, 1, x_264); +lean_ctor_set(x_266, 2, x_263); +lean_ctor_set(x_266, 3, x_265); +x_267 = l_Lean_mkIdentFrom(x_233, x_235, x_238); +lean_dec(x_233); +lean_inc(x_239); +x_268 = l_Lean_Syntax_node2(x_239, x_248, x_254, x_267); +x_269 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__12; +x_270 = l_Lean_Syntax_node2(x_239, x_269, x_266, x_268); +if (lean_is_scalar(x_231)) { + x_271 = lean_alloc_ctor(1, 1, 0); +} else { + x_271 = x_231; +} +lean_ctor_set(x_271, 0, x_270); +x_272 = lean_box(0); +x_273 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_273, 0, x_271); +lean_ctor_set(x_273, 1, x_272); +x_274 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__18; +if (lean_is_scalar(x_259)) { + x_275 = lean_alloc_ctor(0, 2, 0); +} else { + x_275 = x_259; +} +lean_ctor_set(x_275, 0, x_274); +lean_ctor_set(x_275, 1, x_273); +x_276 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__1(x_1, x_2, x_3, x_4, x_5, x_275, x_7, x_8, x_9, x_10, x_11, x_12, x_258); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +return x_276; } -static lean_object* _init_l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___closed__1() { -_start: +else +{ +lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; +lean_dec(x_233); +lean_dec(x_231); +lean_dec(x_230); +lean_dec(x_208); +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_3); +lean_dec(x_2); +x_277 = lean_ctor_get(x_234, 0); +lean_inc(x_277); +x_278 = lean_ctor_get(x_234, 1); +lean_inc(x_278); +if (lean_is_exclusive(x_234)) { + lean_ctor_release(x_234, 0); + lean_ctor_release(x_234, 1); + x_279 = x_234; +} else { + lean_dec_ref(x_234); + 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_211); +x_281 = lean_box(0); +x_282 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_282, 0, x_209); +lean_ctor_set(x_282, 1, x_281); +x_283 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_283, 0, x_208); +lean_ctor_set(x_283, 1, x_282); +x_284 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__1(x_1, x_2, x_3, x_4, x_5, x_283, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +return x_284; +} +} +} +} +} +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__1() { +_start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("invalid use of 'noncomputable' in constructor declaration", 57, 57); +x_1 = lean_mk_string_unchecked("invalid 'protected' field in a 'private' structure", 50, 50); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___closed__2() { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___closed__1; +x_1 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { -uint8_t x_9; -x_9 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 1); -if (x_9 == 0) +uint8_t x_15; +x_15 = l_Lean_Elab_Modifiers_isProtected(x_5); +if (x_15 == 0) { -lean_object* x_10; lean_object* x_11; -x_10 = lean_box(0); -x_11 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__3(x_1, x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -return x_11; +lean_object* x_16; lean_object* x_17; +x_16 = lean_box(0); +x_17 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2(x_1, x_2, x_3, x_4, x_5, x_16, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +return x_17; } else { -lean_object* x_12; lean_object* x_13; uint8_t x_14; -x_12 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___closed__2; -x_13 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -x_14 = !lean_is_exclusive(x_13); -if (x_14 == 0) +uint8_t x_18; +x_18 = l_Lean_Elab_Modifiers_isPrivate(x_6); +if (x_18 == 0) { -return x_13; +lean_object* x_19; lean_object* x_20; +x_19 = lean_box(0); +x_20 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2(x_1, x_2, x_3, x_4, x_5, x_19, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +return x_20; } else { -lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = lean_ctor_get(x_13, 0); -x_16 = lean_ctor_get(x_13, 1); -lean_inc(x_16); -lean_inc(x_15); +lean_object* x_21; lean_object* x_22; uint8_t x_23; +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +x_21 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__2; +x_22 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_21, x_8, x_9, x_10, x_11, x_12, x_13, x_14); lean_dec(x_13); -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_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +x_23 = !lean_is_exclusive(x_22); +if (x_23 == 0) +{ +return x_22; +} +else +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_22, 0); +x_25 = lean_ctor_get(x_22, 1); +lean_inc(x_25); +lean_inc(x_24); +lean_dec(x_22); +x_26 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_26, 0, x_24); +lean_ctor_set(x_26, 1, x_25); +return x_26; +} } } } } -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__19(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4___closed__1() { _start: { -lean_object* x_9; uint8_t x_10; lean_object* x_11; lean_object* x_12; -x_9 = lean_ctor_get(x_6, 1); -lean_inc(x_9); -lean_dec(x_6); -x_10 = 0; -x_11 = l_Lean_Syntax_getPos_x3f(x_1, x_10); -x_12 = l_Lean_Syntax_getTailPos_x3f(x_1, x_10); -if (lean_obj_tag(x_11) == 0) +lean_object* x_1; +x_1 = lean_mk_string_unchecked("invalid 'private' field in a 'private' structure", 48, 48); +return x_1; +} +} +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: { lean_object* x_13; lean_object* x_14; lean_object* x_15; x_13 = lean_unsigned_to_nat(0u); -lean_inc(x_9); -x_14 = l_Lean_FileMap_toPosition(x_9, x_13); -lean_inc(x_14); -x_15 = l_Lean_FileMap_leanPosToLspPos(x_9, x_14); -if (lean_obj_tag(x_12) == 0) -{ -uint8_t x_16; -lean_dec(x_9); -x_16 = !lean_is_exclusive(x_15); -if (x_16 == 0) +x_14 = l_Lean_Syntax_getArg(x_1, x_13); +lean_inc(x_10); +lean_inc(x_6); +x_15 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6(x_14, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_15) == 0) { -lean_object* x_17; lean_object* x_18; lean_object* x_19; +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); x_17 = lean_ctor_get(x_15, 1); -x_18 = lean_ctor_get(x_15, 0); -lean_dec(x_18); lean_inc(x_17); -lean_inc(x_14); -x_19 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_19, 0, x_14); -lean_ctor_set(x_19, 1, x_17); -lean_ctor_set(x_19, 2, x_14); -lean_ctor_set(x_19, 3, x_17); -lean_ctor_set(x_15, 1, x_8); -lean_ctor_set(x_15, 0, x_19); -return x_15; -} -else -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_15, 1); -lean_inc(x_20); lean_dec(x_15); -lean_inc(x_20); -lean_inc(x_14); -x_21 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_21, 0, x_14); -lean_ctor_set(x_21, 1, x_20); -lean_ctor_set(x_21, 2, x_14); -lean_ctor_set(x_21, 3, x_20); -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_21); -lean_ctor_set(x_22, 1, x_8); +lean_inc(x_6); +x_18 = l_Lean_Elab_Command_checkValidFieldModifier(x_16, x_6, x_7, x_8, x_9, x_10, x_11, x_17); +if (lean_obj_tag(x_18) == 0) +{ +lean_object* x_19; uint8_t x_20; +x_19 = lean_ctor_get(x_18, 1); +lean_inc(x_19); +lean_dec(x_18); +x_20 = l_Lean_Elab_Modifiers_isPrivate(x_16); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; +x_21 = lean_box(0); +x_22 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3(x_1, x_2, x_3, x_5, x_16, x_4, x_21, x_6, x_7, x_8, x_9, x_10, x_11, x_19); return x_22; } -} else { uint8_t x_23; -x_23 = !lean_is_exclusive(x_15); +x_23 = l_Lean_Elab_Modifiers_isPrivate(x_4); if (x_23 == 0) { -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_24 = lean_ctor_get(x_15, 1); -x_25 = lean_ctor_get(x_15, 0); -lean_dec(x_25); -x_26 = lean_ctor_get(x_12, 0); -lean_inc(x_26); -lean_dec(x_12); -lean_inc(x_9); -x_27 = l_Lean_FileMap_toPosition(x_9, x_26); -lean_dec(x_26); -lean_inc(x_27); -x_28 = l_Lean_FileMap_leanPosToLspPos(x_9, x_27); -lean_dec(x_9); -x_29 = lean_ctor_get(x_28, 1); -lean_inc(x_29); -lean_dec(x_28); -x_30 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_30, 0, x_14); -lean_ctor_set(x_30, 1, x_24); -lean_ctor_set(x_30, 2, x_27); -lean_ctor_set(x_30, 3, x_29); -lean_ctor_set(x_15, 1, x_8); -lean_ctor_set(x_15, 0, x_30); -return x_15; +lean_object* x_24; lean_object* x_25; +x_24 = lean_box(0); +x_25 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3(x_1, x_2, x_3, x_5, x_16, x_4, x_24, x_6, x_7, x_8, x_9, x_10, x_11, x_19); +return x_25; } else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_31 = lean_ctor_get(x_15, 1); -lean_inc(x_31); -lean_dec(x_15); -x_32 = lean_ctor_get(x_12, 0); -lean_inc(x_32); -lean_dec(x_12); -lean_inc(x_9); -x_33 = l_Lean_FileMap_toPosition(x_9, x_32); -lean_dec(x_32); -lean_inc(x_33); -x_34 = l_Lean_FileMap_leanPosToLspPos(x_9, x_33); +lean_object* x_26; lean_object* x_27; uint8_t x_28; +lean_dec(x_16); +lean_dec(x_3); +lean_dec(x_2); +x_26 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4___closed__2; +x_27 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_26, x_6, x_7, x_8, x_9, x_10, x_11, x_19); +lean_dec(x_11); +lean_dec(x_10); lean_dec(x_9); -x_35 = lean_ctor_get(x_34, 1); -lean_inc(x_35); -lean_dec(x_34); -x_36 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_36, 0, x_14); -lean_ctor_set(x_36, 1, x_31); -lean_ctor_set(x_36, 2, x_33); -lean_ctor_set(x_36, 3, x_35); -x_37 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_37, 0, x_36); -lean_ctor_set(x_37, 1, x_8); -return x_37; +lean_dec(x_8); +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; lean_object* x_31; +x_29 = lean_ctor_get(x_27, 0); +x_30 = lean_ctor_get(x_27, 1); +lean_inc(x_30); +lean_inc(x_29); +lean_dec(x_27); +x_31 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_31, 0, x_29); +lean_ctor_set(x_31, 1, x_30); +return x_31; +} } } } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_11, 0); -lean_inc(x_38); +uint8_t x_32; +lean_dec(x_16); lean_dec(x_11); -lean_inc(x_9); -x_39 = l_Lean_FileMap_toPosition(x_9, x_38); -lean_dec(x_38); -lean_inc(x_39); -x_40 = l_Lean_FileMap_leanPosToLspPos(x_9, x_39); -if (lean_obj_tag(x_12) == 0) -{ -uint8_t x_41; +lean_dec(x_10); lean_dec(x_9); -x_41 = !lean_is_exclusive(x_40); -if (x_41 == 0) +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_3); +lean_dec(x_2); +x_32 = !lean_is_exclusive(x_18); +if (x_32 == 0) { -lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_ctor_get(x_40, 1); -x_43 = lean_ctor_get(x_40, 0); -lean_dec(x_43); -lean_inc(x_42); -lean_inc(x_39); -x_44 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_44, 0, x_39); -lean_ctor_set(x_44, 1, x_42); -lean_ctor_set(x_44, 2, x_39); -lean_ctor_set(x_44, 3, x_42); -lean_ctor_set(x_40, 1, x_8); -lean_ctor_set(x_40, 0, x_44); -return x_40; +return x_18; } else { -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_40, 1); -lean_inc(x_45); -lean_dec(x_40); -lean_inc(x_45); -lean_inc(x_39); -x_46 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_46, 0, x_39); -lean_ctor_set(x_46, 1, x_45); -lean_ctor_set(x_46, 2, x_39); -lean_ctor_set(x_46, 3, x_45); -x_47 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_47, 0, x_46); -lean_ctor_set(x_47, 1, x_8); -return x_47; +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_18, 0); +x_34 = lean_ctor_get(x_18, 1); +lean_inc(x_34); +lean_inc(x_33); +lean_dec(x_18); +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +return x_35; +} } } else { -uint8_t x_48; -x_48 = !lean_is_exclusive(x_40); -if (x_48 == 0) -{ -lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_49 = lean_ctor_get(x_40, 1); -x_50 = lean_ctor_get(x_40, 0); -lean_dec(x_50); -x_51 = lean_ctor_get(x_12, 0); -lean_inc(x_51); -lean_dec(x_12); -lean_inc(x_9); -x_52 = l_Lean_FileMap_toPosition(x_9, x_51); -lean_dec(x_51); -lean_inc(x_52); -x_53 = l_Lean_FileMap_leanPosToLspPos(x_9, x_52); +uint8_t x_36; +lean_dec(x_11); +lean_dec(x_10); lean_dec(x_9); -x_54 = lean_ctor_get(x_53, 1); -lean_inc(x_54); -lean_dec(x_53); -x_55 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_55, 0, x_39); -lean_ctor_set(x_55, 1, x_49); -lean_ctor_set(x_55, 2, x_52); -lean_ctor_set(x_55, 3, x_54); -lean_ctor_set(x_40, 1, x_8); -lean_ctor_set(x_40, 0, x_55); -return x_40; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_3); +lean_dec(x_2); +x_36 = !lean_is_exclusive(x_15); +if (x_36 == 0) +{ +return x_15; } else { -lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_56 = lean_ctor_get(x_40, 1); -lean_inc(x_56); -lean_dec(x_40); -x_57 = lean_ctor_get(x_12, 0); -lean_inc(x_57); -lean_dec(x_12); -lean_inc(x_9); -x_58 = l_Lean_FileMap_toPosition(x_9, x_57); -lean_dec(x_57); -lean_inc(x_58); -x_59 = l_Lean_FileMap_leanPosToLspPos(x_9, x_58); -lean_dec(x_9); -x_60 = lean_ctor_get(x_59, 1); -lean_inc(x_60); -lean_dec(x_59); -x_61 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_61, 0, x_39); -lean_ctor_set(x_61, 1, x_56); -lean_ctor_set(x_61, 2, x_58); -lean_ctor_set(x_61, 3, x_60); -x_62 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_62, 0, x_61); -lean_ctor_set(x_62, 1, x_8); -return x_62; -} +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_15, 0); +x_38 = lean_ctor_get(x_15, 1); +lean_inc(x_38); +lean_inc(x_37); +lean_dec(x_15); +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; } } } } -static lean_object* _init_l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__1() { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__1() { _start: { lean_object* x_1; -x_1 = l_Lean_declRangeExt; +x_1 = lean_mk_string_unchecked("structExplicitBinder", 20, 20); return x_1; } } -static lean_object* _init_l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__2() { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__6; +x_2 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__1; +x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__8; +x_4 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__1; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__3() { _start: { lean_object* x_1; -x_1 = l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_box(0), lean_box(0)); +x_1 = lean_mk_string_unchecked("structImplicitBinder", 20, 20); return x_1; } } -static lean_object* _init_l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__3() { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__4() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__2; -x_2 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__6; +x_2 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__1; +x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__8; +x_4 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__3; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; } } -static lean_object* _init_l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__4() { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__5() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__3; -x_2 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_2, 0, x_1); -lean_ctor_set(x_2, 1, x_1); -return x_2; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("structInstBinder", 16, 16); +return x_1; } } -static lean_object* _init_l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__5() { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__6() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__3; -x_2 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_2, 0, x_1); -lean_ctor_set(x_2, 1, x_1); -return x_2; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__6; +x_2 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__1; +x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__8; +x_4 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__5; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; } } -static lean_object* _init_l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__6() { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__7() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__3; -x_2 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_2, 0, x_1); -lean_ctor_set(x_2, 1, x_1); -lean_ctor_set(x_2, 2, x_1); -lean_ctor_set(x_2, 3, x_1); -return x_2; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("unexpected kind of structure field", 34, 34); +return x_1; } } -static lean_object* _init_l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__7() { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___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_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__5; -x_2 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__3; -x_3 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__6; -x_4 = lean_alloc_ctor(0, 7, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_2); -lean_ctor_set(x_4, 3, x_2); -lean_ctor_set(x_4, 4, x_2); -lean_ctor_set(x_4, 5, x_3); -lean_ctor_set(x_4, 6, x_3); -return x_4; +lean_object* x_1; lean_object* x_2; +x_1 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__7; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_10; uint8_t x_11; -x_10 = lean_st_ref_get(x_8, x_9); -x_11 = !lean_is_exclusive(x_10); -if (x_11 == 0) +lean_object* x_13; lean_object* x_14; uint8_t x_15; +lean_inc(x_4); +x_13 = l_Lean_Syntax_getKind(x_4); +x_14 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__2; +x_15 = lean_name_eq(x_13, x_14); +if (x_15 == 0) { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; -x_12 = lean_ctor_get(x_10, 0); -x_13 = lean_ctor_get(x_10, 1); -x_14 = lean_ctor_get(x_12, 0); -lean_inc(x_14); -lean_dec(x_12); -x_15 = l_Lean_instInhabitedDeclarationRanges; -x_16 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__1; -lean_inc(x_1); -x_17 = l_Lean_MapDeclarationExtension_contains___rarg(x_15, x_16, x_14, x_1); -lean_dec(x_14); +lean_object* x_16; uint8_t x_17; +x_16 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__4; +x_17 = lean_name_eq(x_13, x_16); if (x_17 == 0) { -lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; -lean_free_object(x_10); -x_18 = lean_st_ref_take(x_8, 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 = !lean_is_exclusive(x_19); -if (x_21 == 0) -{ -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; -x_22 = lean_ctor_get(x_19, 0); -x_23 = lean_ctor_get(x_19, 4); -lean_dec(x_23); -x_24 = l_Lean_MapDeclarationExtension_insert___rarg(x_16, x_22, x_1, x_2); -x_25 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__4; -lean_ctor_set(x_19, 4, x_25); -lean_ctor_set(x_19, 0, x_24); -x_26 = lean_st_ref_set(x_8, x_19, x_20); -x_27 = lean_ctor_get(x_26, 1); -lean_inc(x_27); -lean_dec(x_26); -x_28 = lean_st_ref_take(x_6, x_27); -x_29 = lean_ctor_get(x_28, 0); -lean_inc(x_29); -x_30 = lean_ctor_get(x_28, 1); -lean_inc(x_30); -lean_dec(x_28); -x_31 = !lean_is_exclusive(x_29); -if (x_31 == 0) +lean_object* x_18; uint8_t x_19; +x_18 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__6; +x_19 = lean_name_eq(x_13, x_18); +lean_dec(x_13); +if (x_19 == 0) { -lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; -x_32 = lean_ctor_get(x_29, 1); -lean_dec(x_32); -x_33 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__7; -lean_ctor_set(x_29, 1, x_33); -x_34 = lean_st_ref_set(x_6, x_29, x_30); -x_35 = !lean_is_exclusive(x_34); -if (x_35 == 0) +lean_object* x_20; lean_object* x_21; uint8_t x_22; +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_20 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__8; +x_21 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__4(x_20, 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); +x_22 = !lean_is_exclusive(x_21); +if (x_22 == 0) { -lean_object* x_36; lean_object* x_37; -x_36 = lean_ctor_get(x_34, 0); -lean_dec(x_36); -x_37 = lean_box(0); -lean_ctor_set(x_34, 0, x_37); -return x_34; +return x_21; } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_34, 1); -lean_inc(x_38); -lean_dec(x_34); -x_39 = lean_box(0); -x_40 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_40, 0, x_39); -lean_ctor_set(x_40, 1, x_38); -return x_40; +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_21, 0); +x_24 = lean_ctor_get(x_21, 1); +lean_inc(x_24); +lean_inc(x_23); +lean_dec(x_21); +x_25 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +return x_25; } } else { -lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_41 = lean_ctor_get(x_29, 0); -x_42 = lean_ctor_get(x_29, 2); -x_43 = lean_ctor_get(x_29, 3); -x_44 = lean_ctor_get(x_29, 4); -lean_inc(x_44); -lean_inc(x_43); -lean_inc(x_42); -lean_inc(x_41); -lean_dec(x_29); -x_45 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__7; -x_46 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_46, 0, x_41); -lean_ctor_set(x_46, 1, x_45); -lean_ctor_set(x_46, 2, x_42); -lean_ctor_set(x_46, 3, x_43); -lean_ctor_set(x_46, 4, x_44); -x_47 = lean_st_ref_set(x_6, x_46, x_30); -x_48 = lean_ctor_get(x_47, 1); -lean_inc(x_48); -if (lean_is_exclusive(x_47)) { - lean_ctor_release(x_47, 0); - lean_ctor_release(x_47, 1); - x_49 = x_47; -} else { - lean_dec_ref(x_47); - x_49 = lean_box(0); +uint8_t x_26; lean_object* x_27; +x_26 = 3; +x_27 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4(x_4, x_1, x_2, x_3, x_26, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_4); +return x_27; } -x_50 = lean_box(0); -if (lean_is_scalar(x_49)) { - x_51 = lean_alloc_ctor(0, 2, 0); -} else { - x_51 = x_49; } -lean_ctor_set(x_51, 0, x_50); -lean_ctor_set(x_51, 1, x_48); -return x_51; +else +{ +uint8_t x_28; lean_object* x_29; +lean_dec(x_13); +x_28 = 1; +x_29 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4(x_4, x_1, x_2, x_3, x_28, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_4); +return x_29; } } else { -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_52 = lean_ctor_get(x_19, 0); -x_53 = lean_ctor_get(x_19, 1); -x_54 = lean_ctor_get(x_19, 2); -x_55 = lean_ctor_get(x_19, 3); -x_56 = lean_ctor_get(x_19, 5); -x_57 = lean_ctor_get(x_19, 6); -lean_inc(x_57); -lean_inc(x_56); -lean_inc(x_55); -lean_inc(x_54); -lean_inc(x_53); -lean_inc(x_52); -lean_dec(x_19); -x_58 = l_Lean_MapDeclarationExtension_insert___rarg(x_16, x_52, x_1, x_2); -x_59 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__4; -x_60 = lean_alloc_ctor(0, 7, 0); -lean_ctor_set(x_60, 0, x_58); -lean_ctor_set(x_60, 1, x_53); -lean_ctor_set(x_60, 2, x_54); -lean_ctor_set(x_60, 3, x_55); -lean_ctor_set(x_60, 4, x_59); -lean_ctor_set(x_60, 5, x_56); -lean_ctor_set(x_60, 6, x_57); -x_61 = lean_st_ref_set(x_8, x_60, x_20); -x_62 = lean_ctor_get(x_61, 1); -lean_inc(x_62); -lean_dec(x_61); -x_63 = lean_st_ref_take(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); -x_67 = lean_ctor_get(x_64, 2); -lean_inc(x_67); -x_68 = lean_ctor_get(x_64, 3); -lean_inc(x_68); -x_69 = lean_ctor_get(x_64, 4); -lean_inc(x_69); -if (lean_is_exclusive(x_64)) { - lean_ctor_release(x_64, 0); - lean_ctor_release(x_64, 1); - lean_ctor_release(x_64, 2); - lean_ctor_release(x_64, 3); - lean_ctor_release(x_64, 4); - x_70 = x_64; -} else { - lean_dec_ref(x_64); - x_70 = lean_box(0); -} -x_71 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__7; -if (lean_is_scalar(x_70)) { - x_72 = lean_alloc_ctor(0, 5, 0); -} else { - x_72 = x_70; -} -lean_ctor_set(x_72, 0, x_66); -lean_ctor_set(x_72, 1, x_71); -lean_ctor_set(x_72, 2, x_67); -lean_ctor_set(x_72, 3, x_68); -lean_ctor_set(x_72, 4, x_69); -x_73 = lean_st_ref_set(x_6, x_72, x_65); -x_74 = lean_ctor_get(x_73, 1); -lean_inc(x_74); -if (lean_is_exclusive(x_73)) { - lean_ctor_release(x_73, 0); - lean_ctor_release(x_73, 1); - x_75 = x_73; -} else { - lean_dec_ref(x_73); - x_75 = lean_box(0); -} -x_76 = lean_box(0); -if (lean_is_scalar(x_75)) { - x_77 = lean_alloc_ctor(0, 2, 0); -} else { - x_77 = x_75; +uint8_t x_30; lean_object* x_31; +lean_dec(x_13); +x_30 = 0; +x_31 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4(x_4, x_1, x_2, x_3, x_30, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_4); +return x_31; } -lean_ctor_set(x_77, 0, x_76); -lean_ctor_set(x_77, 1, x_74); -return x_77; } } -else +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__1() { +_start: { -lean_object* x_78; -lean_dec(x_2); -lean_dec(x_1); -x_78 = lean_box(0); -lean_ctor_set(x_10, 0, x_78); -return x_10; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("structSimpleBinder", 18, 18); +return x_1; } } -else -{ -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_79 = lean_ctor_get(x_10, 0); -x_80 = lean_ctor_get(x_10, 1); -lean_inc(x_80); -lean_inc(x_79); -lean_dec(x_10); -x_81 = lean_ctor_get(x_79, 0); -lean_inc(x_81); -lean_dec(x_79); -x_82 = l_Lean_instInhabitedDeclarationRanges; -x_83 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__1; -lean_inc(x_1); -x_84 = l_Lean_MapDeclarationExtension_contains___rarg(x_82, x_83, x_81, x_1); -lean_dec(x_81); -if (x_84 == 0) +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__2() { +_start: { -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; -x_85 = lean_st_ref_take(x_8, x_80); -x_86 = lean_ctor_get(x_85, 0); -lean_inc(x_86); -x_87 = lean_ctor_get(x_85, 1); -lean_inc(x_87); -lean_dec(x_85); -x_88 = lean_ctor_get(x_86, 0); -lean_inc(x_88); -x_89 = lean_ctor_get(x_86, 1); -lean_inc(x_89); -x_90 = lean_ctor_get(x_86, 2); -lean_inc(x_90); -x_91 = lean_ctor_get(x_86, 3); -lean_inc(x_91); -x_92 = lean_ctor_get(x_86, 5); -lean_inc(x_92); -x_93 = lean_ctor_get(x_86, 6); -lean_inc(x_93); -if (lean_is_exclusive(x_86)) { - lean_ctor_release(x_86, 0); - lean_ctor_release(x_86, 1); - lean_ctor_release(x_86, 2); - lean_ctor_release(x_86, 3); - lean_ctor_release(x_86, 4); - lean_ctor_release(x_86, 5); - lean_ctor_release(x_86, 6); - x_94 = x_86; -} else { - lean_dec_ref(x_86); - x_94 = lean_box(0); -} -x_95 = l_Lean_MapDeclarationExtension_insert___rarg(x_83, x_88, x_1, x_2); -x_96 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__4; -if (lean_is_scalar(x_94)) { - x_97 = lean_alloc_ctor(0, 7, 0); -} else { - x_97 = x_94; -} -lean_ctor_set(x_97, 0, x_95); -lean_ctor_set(x_97, 1, x_89); -lean_ctor_set(x_97, 2, x_90); -lean_ctor_set(x_97, 3, x_91); -lean_ctor_set(x_97, 4, x_96); -lean_ctor_set(x_97, 5, x_92); -lean_ctor_set(x_97, 6, x_93); -x_98 = lean_st_ref_set(x_8, x_97, x_87); -x_99 = lean_ctor_get(x_98, 1); -lean_inc(x_99); -lean_dec(x_98); -x_100 = lean_st_ref_take(x_6, 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; -} else { - lean_dec_ref(x_101); - x_107 = lean_box(0); -} -x_108 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__7; -if (lean_is_scalar(x_107)) { - x_109 = lean_alloc_ctor(0, 5, 0); -} else { - x_109 = x_107; -} -lean_ctor_set(x_109, 0, x_103); -lean_ctor_set(x_109, 1, x_108); -lean_ctor_set(x_109, 2, x_104); -lean_ctor_set(x_109, 3, x_105); -lean_ctor_set(x_109, 4, x_106); -x_110 = lean_st_ref_set(x_6, x_109, x_102); -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_110); - x_112 = lean_box(0); -} -x_113 = lean_box(0); -if (lean_is_scalar(x_112)) { - x_114 = lean_alloc_ctor(0, 2, 0); -} else { - x_114 = x_112; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__6; +x_2 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__1; +x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__8; +x_4 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__1; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; } -lean_ctor_set(x_114, 0, x_113); -lean_ctor_set(x_114, 1, x_111); -return x_114; } -else +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__3() { +_start: { -lean_object* x_115; lean_object* x_116; -lean_dec(x_2); -lean_dec(x_1); -x_115 = lean_box(0); -x_116 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_116, 0, x_115); -lean_ctor_set(x_116, 1, x_80); -return x_116; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("(", 1, 1); +return x_1; } } +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(")", 1, 1); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__18(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5(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_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; -lean_inc(x_8); -x_11 = l_Lean_Elab_getDeclarationRange___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__19(x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -x_12 = lean_ctor_get(x_11, 0); +uint8_t x_14; +x_14 = lean_usize_dec_eq(x_4, x_5); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; lean_object* x_31; uint8_t x_32; lean_object* x_33; lean_object* x_34; +x_15 = lean_array_uget(x_3, x_4); +lean_inc(x_15); +x_16 = l_Lean_Syntax_getKind(x_15); +x_17 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__2; +x_18 = lean_name_eq(x_16, x_17); +lean_dec(x_16); +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 = lean_ctor_get_uint8(x_11, sizeof(void*)*12); +x_31 = lean_ctor_get(x_11, 11); +x_32 = lean_ctor_get_uint8(x_11, sizeof(void*)*12 + 1); +x_33 = l_Lean_replaceRef(x_15, x_24); +lean_inc(x_31); +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_34 = lean_alloc_ctor(0, 12, 2); +lean_ctor_set(x_34, 0, x_19); +lean_ctor_set(x_34, 1, x_20); +lean_ctor_set(x_34, 2, x_21); +lean_ctor_set(x_34, 3, x_22); +lean_ctor_set(x_34, 4, x_23); +lean_ctor_set(x_34, 5, x_33); +lean_ctor_set(x_34, 6, x_25); +lean_ctor_set(x_34, 7, x_26); +lean_ctor_set(x_34, 8, x_27); +lean_ctor_set(x_34, 9, x_28); +lean_ctor_set(x_34, 10, x_29); +lean_ctor_set(x_34, 11, x_31); +lean_ctor_set_uint8(x_34, sizeof(void*)*12, x_30); +lean_ctor_set_uint8(x_34, sizeof(void*)*12 + 1, x_32); +if (x_18 == 0) +{ +lean_object* x_35; lean_object* x_36; +x_35 = lean_box(0); lean_inc(x_12); -x_13 = lean_ctor_get(x_11, 1); -lean_inc(x_13); -lean_dec(x_11); +lean_inc(x_10); +lean_inc(x_9); lean_inc(x_8); -x_14 = l_Lean_Elab_getDeclarationRange___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__19(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); -x_15 = !lean_is_exclusive(x_14); -if (x_15 == 0) +lean_inc(x_7); +lean_inc(x_2); +x_36 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5(x_6, x_2, x_1, x_15, x_35, x_7, x_8, x_9, x_10, x_34, x_12, x_13); +if (lean_obj_tag(x_36) == 0) { -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_14, 0); -x_17 = lean_ctor_get(x_14, 1); -lean_ctor_set(x_14, 1, x_16); -lean_ctor_set(x_14, 0, x_12); -x_18 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20(x_1, x_14, x_4, x_5, x_6, x_7, x_8, x_9, x_17); -lean_dec(x_8); -return x_18; +lean_object* x_37; lean_object* x_38; size_t x_39; size_t x_40; +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 = 1; +x_40 = lean_usize_add(x_4, x_39); +x_4 = x_40; +x_6 = x_37; +x_13 = x_38; +goto _start; } else { -lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_19 = lean_ctor_get(x_14, 0); -x_20 = lean_ctor_get(x_14, 1); -lean_inc(x_20); -lean_inc(x_19); -lean_dec(x_14); -x_21 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_21, 0, x_12); -lean_ctor_set(x_21, 1, x_19); -x_22 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20(x_1, x_21, x_4, x_5, x_6, x_7, x_8, x_9, x_20); +uint8_t x_42; +lean_dec(x_12); +lean_dec(x_10); +lean_dec(x_9); lean_dec(x_8); -return x_22; +lean_dec(x_7); +lean_dec(x_2); +x_42 = !lean_is_exclusive(x_36); +if (x_42 == 0) +{ +return x_36; +} +else +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_36, 0); +x_44 = lean_ctor_get(x_36, 1); +lean_inc(x_44); +lean_inc(x_43); +lean_dec(x_36); +x_45 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_45, 0, x_43); +lean_ctor_set(x_45, 1, x_44); +return x_45; } } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; lean_object* x_17; -x_12 = lean_unsigned_to_nat(1u); -x_13 = l_Lean_Syntax_getArg(x_1, x_12); -x_14 = l_Lean_Syntax_getId(x_13); -lean_inc(x_14); -x_15 = l_Lean_Name_append(x_2, x_14); -x_16 = lean_ctor_get_uint8(x_3, sizeof(void*)*2); -lean_inc(x_5); -x_17 = l_Lean_Elab_applyVisibility___at_Lean_Elab_Term_expandDeclId___spec__5(x_16, x_15, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_17) == 0) +else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_17, 1); -lean_inc(x_19); -lean_dec(x_17); -x_20 = lean_ctor_get(x_3, 0); -lean_inc(x_20); -lean_inc(x_5); -lean_inc(x_18); -x_21 = l_Lean_addDocString_x27___at_Lean_Elab_Term_expandDeclId___spec__8(x_18, x_20, x_5, x_6, x_7, x_8, x_9, x_10, x_19); -if (lean_obj_tag(x_21) == 0) -{ -lean_object* x_22; lean_object* x_23; uint8_t x_24; -x_22 = lean_ctor_get(x_21, 1); -lean_inc(x_22); -lean_dec(x_21); -lean_inc(x_18); -x_23 = l_Lean_Elab_addAuxDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__18(x_18, x_13, x_13, x_5, x_6, x_7, x_8, x_9, x_10, x_22); -lean_dec(x_5); -x_24 = !lean_is_exclusive(x_23); -if (x_24 == 0) -{ -lean_object* x_25; lean_object* x_26; -x_25 = lean_ctor_get(x_23, 0); -lean_dec(x_25); -x_26 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_26, 0, x_13); -lean_ctor_set(x_26, 1, x_3); -lean_ctor_set(x_26, 2, x_14); -lean_ctor_set(x_26, 3, x_18); -lean_ctor_set(x_23, 0, x_26); -return x_23; -} -else +lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; +x_46 = lean_unsigned_to_nat(0u); +x_47 = l_Lean_Syntax_getArg(x_15, x_46); +x_48 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__3; +x_49 = 0; +x_50 = l_Lean_mkAtomFrom(x_15, x_48, x_49); +x_51 = lean_unsigned_to_nat(1u); +x_52 = l_Lean_Syntax_getArg(x_15, x_51); +x_53 = lean_box(0); +x_54 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_54, 0, x_52); +lean_ctor_set(x_54, 1, x_53); +x_55 = lean_array_mk(x_54); +x_56 = lean_box(2); +x_57 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__10; +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_unsigned_to_nat(2u); +x_60 = l_Lean_Syntax_getArg(x_15, x_59); +x_61 = lean_unsigned_to_nat(3u); +x_62 = l_Lean_Syntax_getArg(x_15, x_61); +x_63 = lean_unsigned_to_nat(4u); +x_64 = l_Lean_Syntax_getArg(x_15, x_63); +x_65 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__4; +x_66 = l_Lean_mkAtomFrom(x_15, x_65, x_49); +lean_dec(x_15); +x_67 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_67, 0, x_66); +lean_ctor_set(x_67, 1, x_53); +x_68 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_68, 0, x_64); +lean_ctor_set(x_68, 1, x_67); +x_69 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_69, 0, x_62); +lean_ctor_set(x_69, 1, x_68); +x_70 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_70, 0, x_60); +lean_ctor_set(x_70, 1, x_69); +x_71 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_71, 0, x_58); +lean_ctor_set(x_71, 1, x_70); +x_72 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_72, 0, x_50); +lean_ctor_set(x_72, 1, x_71); +x_73 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_73, 0, x_47); +lean_ctor_set(x_73, 1, x_72); +x_74 = lean_array_mk(x_73); +x_75 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__2; +x_76 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_76, 0, x_56); +lean_ctor_set(x_76, 1, x_75); +lean_ctor_set(x_76, 2, x_74); +x_77 = lean_box(0); +lean_inc(x_12); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_2); +x_78 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5(x_6, x_2, x_1, x_76, x_77, x_7, x_8, x_9, x_10, x_34, x_12, x_13); +if (lean_obj_tag(x_78) == 0) { -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_alloc_ctor(0, 4, 0); -lean_ctor_set(x_28, 0, x_13); -lean_ctor_set(x_28, 1, x_3); -lean_ctor_set(x_28, 2, x_14); -lean_ctor_set(x_28, 3, x_18); -x_29 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_29, 0, x_28); -lean_ctor_set(x_29, 1, x_27); -return x_29; -} +lean_object* x_79; lean_object* x_80; size_t x_81; size_t x_82; +x_79 = lean_ctor_get(x_78, 0); +lean_inc(x_79); +x_80 = lean_ctor_get(x_78, 1); +lean_inc(x_80); +lean_dec(x_78); +x_81 = 1; +x_82 = lean_usize_add(x_4, x_81); +x_4 = x_82; +x_6 = x_79; +x_13 = x_80; +goto _start; } else { -uint8_t x_30; -lean_dec(x_18); -lean_dec(x_14); -lean_dec(x_13); +uint8_t x_84; +lean_dec(x_12); +lean_dec(x_10); lean_dec(x_9); -lean_dec(x_5); -lean_dec(x_3); -x_30 = !lean_is_exclusive(x_21); -if (x_30 == 0) +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_2); +x_84 = !lean_is_exclusive(x_78); +if (x_84 == 0) { -return x_21; +return x_78; } else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_31 = lean_ctor_get(x_21, 0); -x_32 = lean_ctor_get(x_21, 1); -lean_inc(x_32); -lean_inc(x_31); -lean_dec(x_21); -x_33 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_33, 0, x_31); -lean_ctor_set(x_33, 1, x_32); -return x_33; +lean_object* x_85; lean_object* x_86; lean_object* x_87; +x_85 = lean_ctor_get(x_78, 0); +x_86 = lean_ctor_get(x_78, 1); +lean_inc(x_86); +lean_inc(x_85); +lean_dec(x_78); +x_87 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_87, 0, x_85); +lean_ctor_set(x_87, 1, x_86); +return x_87; } } } -else -{ -uint8_t x_34; -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_9); -lean_dec(x_5); -lean_dec(x_3); -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; -} -} -} -} -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__2___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("invalid 'protected' constructor in a 'private' structure", 56, 56); -return x_1; -} +lean_object* x_88; +lean_dec(x_12); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_2); +x_88 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_88, 0, x_6); +lean_ctor_set(x_88, 1, x_13); +return x_88; } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__2___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__2___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___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: { -uint8_t x_13; -x_13 = l_Lean_Elab_Modifiers_isProtected(x_3); -if (x_13 == 0) -{ -lean_object* x_14; lean_object* x_15; -x_14 = lean_box(0); -x_15 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__1(x_1, x_2, x_3, x_14, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -return x_15; -} -else -{ -uint8_t x_16; -x_16 = l_Lean_Elab_Modifiers_isPrivate(x_4); -if (x_16 == 0) -{ -lean_object* x_17; lean_object* x_18; -x_17 = lean_box(0); -x_18 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__1(x_1, x_2, x_3, x_17, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -return x_18; -} -else -{ -lean_object* x_19; lean_object* x_20; uint8_t x_21; -lean_dec(x_3); -lean_dec(x_2); -x_19 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__2___closed__2; -x_20 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_19, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_10); -x_21 = !lean_is_exclusive(x_20); -if (x_21 == 0) -{ -return x_20; -} -else +uint8_t x_14; +x_14 = lean_usize_dec_eq(x_4, x_5); +if (x_14 == 0) { -lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_22 = lean_ctor_get(x_20, 0); -x_23 = lean_ctor_get(x_20, 1); +lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; lean_object* x_31; uint8_t x_32; lean_object* x_33; lean_object* x_34; +x_15 = lean_array_uget(x_3, x_4); +lean_inc(x_15); +x_16 = l_Lean_Syntax_getKind(x_15); +x_17 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__2; +x_18 = lean_name_eq(x_16, x_17); +lean_dec(x_16); +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 = lean_ctor_get_uint8(x_11, sizeof(void*)*12); +x_31 = lean_ctor_get(x_11, 11); +x_32 = lean_ctor_get_uint8(x_11, sizeof(void*)*12 + 1); +x_33 = l_Lean_replaceRef(x_15, x_24); +lean_inc(x_31); +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_dec(x_20); -x_24 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_24, 0, x_22); -lean_ctor_set(x_24, 1, x_23); -return x_24; +lean_inc(x_21); +lean_inc(x_20); +lean_inc(x_19); +x_34 = lean_alloc_ctor(0, 12, 2); +lean_ctor_set(x_34, 0, x_19); +lean_ctor_set(x_34, 1, x_20); +lean_ctor_set(x_34, 2, x_21); +lean_ctor_set(x_34, 3, x_22); +lean_ctor_set(x_34, 4, x_23); +lean_ctor_set(x_34, 5, x_33); +lean_ctor_set(x_34, 6, x_25); +lean_ctor_set(x_34, 7, x_26); +lean_ctor_set(x_34, 8, x_27); +lean_ctor_set(x_34, 9, x_28); +lean_ctor_set(x_34, 10, x_29); +lean_ctor_set(x_34, 11, x_31); +lean_ctor_set_uint8(x_34, sizeof(void*)*12, x_30); +lean_ctor_set_uint8(x_34, sizeof(void*)*12 + 1, x_32); +if (x_18 == 0) +{ +lean_object* x_35; lean_object* x_36; +x_35 = lean_box(0); +lean_inc(x_12); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_2); +x_36 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5(x_6, x_2, x_1, x_15, x_35, x_7, x_8, x_9, x_10, x_34, x_12, x_13); +if (lean_obj_tag(x_36) == 0) +{ +lean_object* x_37; lean_object* x_38; size_t x_39; size_t x_40; +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 = 1; +x_40 = lean_usize_add(x_4, x_39); +x_4 = x_40; +x_6 = x_37; +x_13 = x_38; +goto _start; } +else +{ +uint8_t x_42; +lean_dec(x_12); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_2); +x_42 = !lean_is_exclusive(x_36); +if (x_42 == 0) +{ +return x_36; } +else +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_36, 0); +x_44 = lean_ctor_get(x_36, 1); +lean_inc(x_44); +lean_inc(x_43); +lean_dec(x_36); +x_45 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_45, 0, x_43); +lean_ctor_set(x_45, 1, x_44); +return x_45; } } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__1() { +else +{ +lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; +x_46 = lean_unsigned_to_nat(0u); +x_47 = l_Lean_Syntax_getArg(x_15, x_46); +x_48 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__3; +x_49 = 0; +x_50 = l_Lean_mkAtomFrom(x_15, x_48, x_49); +x_51 = lean_unsigned_to_nat(1u); +x_52 = l_Lean_Syntax_getArg(x_15, x_51); +x_53 = lean_box(0); +x_54 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_54, 0, x_52); +lean_ctor_set(x_54, 1, x_53); +x_55 = lean_array_mk(x_54); +x_56 = lean_box(2); +x_57 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__10; +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_unsigned_to_nat(2u); +x_60 = l_Lean_Syntax_getArg(x_15, x_59); +x_61 = lean_unsigned_to_nat(3u); +x_62 = l_Lean_Syntax_getArg(x_15, x_61); +x_63 = lean_unsigned_to_nat(4u); +x_64 = l_Lean_Syntax_getArg(x_15, x_63); +x_65 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__4; +x_66 = l_Lean_mkAtomFrom(x_15, x_65, x_49); +lean_dec(x_15); +x_67 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_67, 0, x_66); +lean_ctor_set(x_67, 1, x_53); +x_68 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_68, 0, x_64); +lean_ctor_set(x_68, 1, x_67); +x_69 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_69, 0, x_62); +lean_ctor_set(x_69, 1, x_68); +x_70 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_70, 0, x_60); +lean_ctor_set(x_70, 1, x_69); +x_71 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_71, 0, x_58); +lean_ctor_set(x_71, 1, x_70); +x_72 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_72, 0, x_50); +lean_ctor_set(x_72, 1, x_71); +x_73 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_73, 0, x_47); +lean_ctor_set(x_73, 1, x_72); +x_74 = lean_array_mk(x_73); +x_75 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__2; +x_76 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_76, 0, x_56); +lean_ctor_set(x_76, 1, x_75); +lean_ctor_set(x_76, 2, x_74); +x_77 = lean_box(0); +lean_inc(x_12); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_2); +x_78 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5(x_6, x_2, x_1, x_76, x_77, x_7, x_8, x_9, x_10, x_34, x_12, x_13); +if (lean_obj_tag(x_78) == 0) +{ +lean_object* x_79; lean_object* x_80; size_t x_81; size_t x_82; +x_79 = lean_ctor_get(x_78, 0); +lean_inc(x_79); +x_80 = lean_ctor_get(x_78, 1); +lean_inc(x_80); +lean_dec(x_78); +x_81 = 1; +x_82 = lean_usize_add(x_4, x_81); +x_4 = x_82; +x_6 = x_79; +x_13 = x_80; +goto _start; +} +else +{ +uint8_t x_84; +lean_dec(x_12); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_2); +x_84 = !lean_is_exclusive(x_78); +if (x_84 == 0) +{ +return x_78; +} +else +{ +lean_object* x_85; lean_object* x_86; lean_object* x_87; +x_85 = lean_ctor_get(x_78, 0); +x_86 = lean_ctor_get(x_78, 1); +lean_inc(x_86); +lean_inc(x_85); +lean_dec(x_78); +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_dec(x_12); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_2); +x_88 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_88, 0, x_6); +lean_ctor_set(x_88, 1, x_13); +return x_88; +} +} +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__1() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("invalid 'private' constructor in a 'private' structure", 54, 54); -return x_1; +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_array_mk(x_1); +return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__2() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__1; +x_2 = lean_array_get_size(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__3() { +static uint8_t _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__3() { _start: { -lean_object* x_1; uint8_t x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; -x_1 = lean_box(0); -x_2 = 0; -x_3 = 0; -x_4 = 2; -x_5 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; -x_6 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_6, 0, x_1); -lean_ctor_set(x_6, 1, x_5); -lean_ctor_set_uint8(x_6, sizeof(void*)*2, x_2); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 1, x_3); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 2, x_4); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 3, x_3); -return x_6; +lean_object* x_1; lean_object* x_2; uint8_t x_3; +x_1 = lean_unsigned_to_nat(0u); +x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__2; +x_3 = lean_nat_dec_lt(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +static uint8_t _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___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; uint8_t x_18; -x_11 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_defaultCtorName; -lean_inc(x_3); -x_12 = l_Lean_Name_append(x_3, x_11); -x_13 = lean_unsigned_to_nat(1u); -x_14 = l_Lean_Syntax_getArg(x_1, x_13); -x_15 = l_Lean_Syntax_mkSynthetic(x_14); -x_16 = lean_unsigned_to_nat(5u); -x_17 = l_Lean_Syntax_getArg(x_1, x_16); -x_18 = l_Lean_Syntax_isNone(x_17); -if (x_18 == 0) +lean_object* x_1; uint8_t x_2; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__2; +x_2 = lean_nat_dec_le(x_1, x_1); +return x_2; +} +} +static size_t _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__5() { +_start: { -lean_object* x_19; uint8_t x_20; -x_19 = l_Lean_Syntax_getArg(x_17, x_13); -lean_dec(x_17); -x_20 = l_Lean_Syntax_isNone(x_19); -if (x_20 == 0) +lean_object* x_1; size_t x_2; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__2; +x_2 = lean_usize_of_nat(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___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_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; -lean_dec(x_15); -lean_dec(x_12); -x_21 = lean_unsigned_to_nat(0u); -x_22 = l_Lean_Syntax_getArg(x_19, x_21); -lean_dec(x_19); -x_23 = l_Lean_Syntax_getArg(x_22, x_21); -x_24 = !lean_is_exclusive(x_8); -if (x_24 == 0) +lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_12 = lean_unsigned_to_nat(5u); +x_13 = l_Lean_Syntax_getArg(x_1, x_12); +x_14 = l_Lean_Syntax_isNone(x_13); +if (x_14 == 0) { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_8, 5); -x_26 = l_Lean_replaceRef(x_22, x_25); -lean_dec(x_25); -lean_ctor_set(x_8, 5, x_26); -lean_inc(x_8); -lean_inc(x_4); -x_27 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1(x_23, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_23); -if (lean_obj_tag(x_27) == 0) +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_15 = lean_unsigned_to_nat(2u); +x_16 = l_Lean_Syntax_getArg(x_13, x_15); +lean_dec(x_13); +x_17 = lean_unsigned_to_nat(0u); +x_18 = l_Lean_Syntax_getArg(x_16, x_17); +lean_dec(x_16); +x_19 = l_Lean_Syntax_getArgs(x_18); +lean_dec(x_18); +x_20 = lean_array_get_size(x_19); +x_21 = lean_nat_dec_lt(x_17, x_20); +if (x_21 == 0) { -lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_28 = lean_ctor_get(x_27, 0); -lean_inc(x_28); -x_29 = lean_ctor_get(x_27, 1); -lean_inc(x_29); -lean_dec(x_27); -lean_inc(x_4); -x_30 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17(x_28, x_4, x_5, x_6, x_7, x_8, x_9, x_29); -if (lean_obj_tag(x_30) == 0) +lean_object* x_22; lean_object* x_23; +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +x_22 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__1; +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_11); +return x_23; +} +else { -lean_object* x_31; uint8_t x_32; -x_31 = lean_ctor_get(x_30, 1); -lean_inc(x_31); -lean_dec(x_30); -x_32 = l_Lean_Elab_Modifiers_isPrivate(x_28); -if (x_32 == 0) +uint8_t x_24; +x_24 = lean_nat_dec_le(x_20, x_20); +if (x_24 == 0) { -lean_object* x_33; lean_object* x_34; -x_33 = lean_box(0); -x_34 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__2(x_22, x_3, x_28, x_2, x_33, x_4, x_5, x_6, x_7, x_8, x_9, x_31); -lean_dec(x_22); -return x_34; +lean_object* x_25; lean_object* x_26; +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +x_25 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___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_11); +return x_26; } else { -uint8_t x_35; -x_35 = l_Lean_Elab_Modifiers_isPrivate(x_2); -if (x_35 == 0) -{ -lean_object* x_36; lean_object* x_37; -x_36 = lean_box(0); -x_37 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__2(x_22, x_3, x_28, x_2, x_36, x_4, x_5, x_6, x_7, x_8, x_9, x_31); -lean_dec(x_22); -return x_37; +size_t x_27; size_t x_28; lean_object* x_29; lean_object* x_30; +x_27 = 0; +x_28 = lean_usize_of_nat(x_20); +lean_dec(x_20); +x_29 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__1; +x_30 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5(x_2, x_3, x_19, x_27, x_28, x_29, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_19); +return x_30; +} +} } else { -lean_object* x_38; lean_object* x_39; uint8_t x_40; -lean_dec(x_28); -lean_dec(x_22); -lean_dec(x_3); -x_38 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__2; -x_39 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_38, x_4, x_5, x_6, x_7, x_8, x_9, x_31); +uint8_t x_31; +lean_dec(x_13); +x_31 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__3; +if (x_31 == 0) +{ +lean_object* x_32; lean_object* x_33; +lean_dec(x_10); lean_dec(x_8); -x_40 = !lean_is_exclusive(x_39); -if (x_40 == 0) +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +x_32 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___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_11); +return x_33; +} +else { -return x_39; +uint8_t x_34; +x_34 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__4; +if (x_34 == 0) +{ +lean_object* x_35; lean_object* x_36; +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +x_35 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__1; +x_36 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_36, 0, x_35); +lean_ctor_set(x_36, 1, x_11); +return x_36; } else { -lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_ctor_get(x_39, 0); -x_42 = lean_ctor_get(x_39, 1); -lean_inc(x_42); -lean_inc(x_41); -lean_dec(x_39); -x_43 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_43, 0, x_41); -lean_ctor_set(x_43, 1, x_42); -return x_43; +size_t x_37; lean_object* x_38; size_t x_39; lean_object* x_40; +x_37 = 0; +x_38 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__1; +x_39 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__5; +x_40 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__6(x_2, x_3, x_38, x_37, x_39, x_38, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_40; } } } } -else +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__1() { +_start: { -uint8_t x_44; -lean_dec(x_28); -lean_dec(x_8); -lean_dec(x_22); -lean_dec(x_4); -lean_dec(x_3); -x_44 = !lean_is_exclusive(x_30); -if (x_44 == 0) +lean_object* x_1; +x_1 = lean_mk_string_unchecked(":=", 2, 2); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__2() { +_start: { -return x_30; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("classTk", 7, 7); +return x_1; } -else +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__3() { +_start: { -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_30, 0); -x_46 = lean_ctor_get(x_30, 1); -lean_inc(x_46); -lean_inc(x_45); -lean_dec(x_30); -x_47 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_47, 0, x_45); -lean_ctor_set(x_47, 1, x_46); -return x_47; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__6; +x_2 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__1; +x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__8; +x_4 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__2; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} } +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("structure", 9, 9); +return x_1; } } -else +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__5() { +_start: { -uint8_t x_48; -lean_dec(x_8); -lean_dec(x_22); -lean_dec(x_4); -lean_dec(x_3); -x_48 = !lean_is_exclusive(x_27); -if (x_48 == 0) +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__3; +x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__4; +x_3 = lean_string_append(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__6() { +_start: { -return x_27; +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" ... :=' has been deprecated in favor of '", 42, 42); +return x_1; } -else +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__7() { +_start: { -lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_49 = lean_ctor_get(x_27, 0); -x_50 = lean_ctor_get(x_27, 1); -lean_inc(x_50); -lean_inc(x_49); -lean_dec(x_27); -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_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__5; +x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__6; +x_3 = lean_string_append(x_1, x_2); +return x_3; +} } +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__7; +x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__4; +x_3 = lean_string_append(x_1, x_2); +return x_3; } } -else +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__9() { +_start: { -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; uint8_t x_63; lean_object* x_64; uint8_t x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_52 = lean_ctor_get(x_8, 0); -x_53 = lean_ctor_get(x_8, 1); -x_54 = lean_ctor_get(x_8, 2); -x_55 = lean_ctor_get(x_8, 3); -x_56 = lean_ctor_get(x_8, 4); -x_57 = lean_ctor_get(x_8, 5); -x_58 = lean_ctor_get(x_8, 6); -x_59 = lean_ctor_get(x_8, 7); -x_60 = lean_ctor_get(x_8, 8); -x_61 = lean_ctor_get(x_8, 9); -x_62 = lean_ctor_get(x_8, 10); -x_63 = lean_ctor_get_uint8(x_8, sizeof(void*)*12); -x_64 = lean_ctor_get(x_8, 11); -x_65 = lean_ctor_get_uint8(x_8, sizeof(void*)*12 + 1); -lean_inc(x_64); -lean_inc(x_62); -lean_inc(x_61); -lean_inc(x_60); -lean_inc(x_59); -lean_inc(x_58); -lean_inc(x_57); -lean_inc(x_56); -lean_inc(x_55); -lean_inc(x_54); -lean_inc(x_53); -lean_inc(x_52); -lean_dec(x_8); -x_66 = l_Lean_replaceRef(x_22, x_57); -lean_dec(x_57); -x_67 = lean_alloc_ctor(0, 12, 2); -lean_ctor_set(x_67, 0, x_52); -lean_ctor_set(x_67, 1, x_53); -lean_ctor_set(x_67, 2, x_54); -lean_ctor_set(x_67, 3, x_55); -lean_ctor_set(x_67, 4, x_56); -lean_ctor_set(x_67, 5, x_66); -lean_ctor_set(x_67, 6, x_58); -lean_ctor_set(x_67, 7, x_59); -lean_ctor_set(x_67, 8, x_60); -lean_ctor_set(x_67, 9, x_61); -lean_ctor_set(x_67, 10, x_62); -lean_ctor_set(x_67, 11, x_64); -lean_ctor_set_uint8(x_67, sizeof(void*)*12, x_63); -lean_ctor_set_uint8(x_67, sizeof(void*)*12 + 1, x_65); -lean_inc(x_67); -lean_inc(x_4); -x_68 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1(x_23, x_4, x_5, x_6, x_7, x_67, x_9, x_10); -lean_dec(x_23); -if (lean_obj_tag(x_68) == 0) -{ -lean_object* x_69; lean_object* x_70; lean_object* x_71; -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_4); -x_71 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17(x_69, x_4, x_5, x_6, x_7, x_67, x_9, x_70); -if (lean_obj_tag(x_71) == 0) -{ -lean_object* x_72; uint8_t x_73; -x_72 = lean_ctor_get(x_71, 1); -lean_inc(x_72); -lean_dec(x_71); -x_73 = l_Lean_Elab_Modifiers_isPrivate(x_69); -if (x_73 == 0) -{ -lean_object* x_74; lean_object* x_75; -x_74 = lean_box(0); -x_75 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__2(x_22, x_3, x_69, x_2, x_74, x_4, x_5, x_6, x_7, x_67, x_9, x_72); -lean_dec(x_22); -return x_75; +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" ... where'.", 12, 12); +return x_1; } -else -{ -uint8_t x_76; -x_76 = l_Lean_Elab_Modifiers_isPrivate(x_2); -if (x_76 == 0) -{ -lean_object* x_77; lean_object* x_78; -x_77 = lean_box(0); -x_78 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__2(x_22, x_3, x_69, x_2, x_77, x_4, x_5, x_6, x_7, x_67, x_9, x_72); -lean_dec(x_22); -return x_78; } -else +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__10() { +_start: { -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_69); -lean_dec(x_22); -lean_dec(x_3); -x_79 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__2; -x_80 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_79, x_4, x_5, x_6, x_7, x_67, x_9, x_72); -lean_dec(x_67); -x_81 = lean_ctor_get(x_80, 0); -lean_inc(x_81); -x_82 = lean_ctor_get(x_80, 1); -lean_inc(x_82); -if (lean_is_exclusive(x_80)) { - lean_ctor_release(x_80, 0); - lean_ctor_release(x_80, 1); - x_83 = x_80; -} else { - lean_dec_ref(x_80); - x_83 = lean_box(0); -} -if (lean_is_scalar(x_83)) { - x_84 = lean_alloc_ctor(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; -} +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__8; +x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__9; +x_3 = lean_string_append(x_1, x_2); +return x_3; } } -else +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__11() { +_start: { -lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; -lean_dec(x_69); -lean_dec(x_67); -lean_dec(x_22); -lean_dec(x_4); -lean_dec(x_3); -x_85 = lean_ctor_get(x_71, 0); -lean_inc(x_85); -x_86 = lean_ctor_get(x_71, 1); -lean_inc(x_86); -if (lean_is_exclusive(x_71)) { - lean_ctor_release(x_71, 0); - lean_ctor_release(x_71, 1); - x_87 = x_71; -} else { - lean_dec_ref(x_71); - x_87 = lean_box(0); -} -if (lean_is_scalar(x_87)) { - x_88 = lean_alloc_ctor(1, 2, 0); -} else { - x_88 = x_87; -} -lean_ctor_set(x_88, 0, x_85); -lean_ctor_set(x_88, 1, x_86); -return x_88; +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__10; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; } } -else +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__12() { +_start: { -lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; -lean_dec(x_67); -lean_dec(x_22); -lean_dec(x_4); -lean_dec(x_3); -x_89 = lean_ctor_get(x_68, 0); -lean_inc(x_89); -x_90 = lean_ctor_get(x_68, 1); -lean_inc(x_90); -if (lean_is_exclusive(x_68)) { - lean_ctor_release(x_68, 0); - lean_ctor_release(x_68, 1); - x_91 = x_68; -} else { - lean_dec_ref(x_68); - x_91 = lean_box(0); -} -if (lean_is_scalar(x_91)) { - x_92 = lean_alloc_ctor(1, 2, 0); -} else { - x_92 = x_91; -} -lean_ctor_set(x_92, 0, x_89); -lean_ctor_set(x_92, 1, x_90); -return x_92; -} -} +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__11; +x_2 = l_Lean_MessageData_ofFormat(x_1); +return x_2; } -else -{ -lean_object* x_93; uint8_t x_94; -lean_dec(x_19); -lean_dec(x_3); -lean_inc(x_12); -x_93 = l_Lean_Elab_addAuxDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__18(x_12, x_15, x_15, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_4); -x_94 = !lean_is_exclusive(x_93); -if (x_94 == 0) -{ -lean_object* x_95; lean_object* x_96; lean_object* x_97; -x_95 = lean_ctor_get(x_93, 0); -lean_dec(x_95); -x_96 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__3; -x_97 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_97, 0, x_15); -lean_ctor_set(x_97, 1, x_96); -lean_ctor_set(x_97, 2, x_11); -lean_ctor_set(x_97, 3, x_12); -lean_ctor_set(x_93, 0, x_97); -return x_93; } -else +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__13() { +_start: { -lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; -x_98 = lean_ctor_get(x_93, 1); -lean_inc(x_98); -lean_dec(x_93); -x_99 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__3; -x_100 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_100, 0, x_15); -lean_ctor_set(x_100, 1, x_99); -lean_ctor_set(x_100, 2, x_11); -lean_ctor_set(x_100, 3, x_12); -x_101 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_101, 0, x_100); -lean_ctor_set(x_101, 1, x_98); -return x_101; -} -} +lean_object* x_1; +x_1 = l_Lean_Linter_linter_deprecated; +return x_1; } -else -{ -lean_object* x_102; uint8_t x_103; -lean_dec(x_17); -lean_dec(x_3); -lean_inc(x_12); -x_102 = l_Lean_Elab_addAuxDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__18(x_12, x_15, x_15, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_4); -x_103 = !lean_is_exclusive(x_102); -if (x_103 == 0) -{ -lean_object* x_104; lean_object* x_105; lean_object* x_106; -x_104 = lean_ctor_get(x_102, 0); -lean_dec(x_104); -x_105 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__3; -x_106 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_106, 0, x_15); -lean_ctor_set(x_106, 1, x_105); -lean_ctor_set(x_106, 2, x_11); -lean_ctor_set(x_106, 3, x_12); -lean_ctor_set(x_102, 0, x_106); -return x_102; } -else +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__14() { +_start: { -lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; -x_107 = lean_ctor_get(x_102, 1); -lean_inc(x_107); -lean_dec(x_102); -x_108 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__3; -x_109 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_109, 0, x_15); -lean_ctor_set(x_109, 1, x_108); -lean_ctor_set(x_109, 2, x_11); -lean_ctor_set(x_109, 3, x_12); -x_110 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_110, 0, x_109); -lean_ctor_set(x_110, 1, x_107); -return x_110; -} -} +lean_object* x_1; +x_1 = lean_mk_string_unchecked("class", 5, 5); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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) { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__15() { _start: { -lean_object* x_9; -x_9 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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); -return x_9; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__3; +x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__14; +x_3 = lean_string_append(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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) { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__16() { _start: { -lean_object* x_10; -x_10 = l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__6(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_1); -return x_10; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__15; +x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__6; +x_3 = lean_string_append(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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) { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__17() { _start: { -lean_object* x_9; -x_9 = l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_9; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__16; +x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__14; +x_3 = lean_string_append(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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) { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__18() { _start: { -lean_object* x_7; -x_7 = l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__9(x_1, x_2, x_3, x_4, x_5, x_6); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_7; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__17; +x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__9; +x_3 = lean_string_append(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__5___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__19() { _start: { -lean_object* x_5; -x_5 = l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__5___lambda__1(x_1, x_2, x_3, x_4); -lean_dec(x_3); -lean_dec(x_1); -return x_5; +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___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_Lean_Elab_liftMacroM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__5___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__20() { _start: { -lean_object* x_5; -x_5 = l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__5___lambda__2(x_1, x_2, x_3, x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_5; +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__19; +x_2 = l_Lean_MessageData_ofFormat(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__5___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___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_7; -x_7 = l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__5___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6); -lean_dec(x_5); -lean_dec(x_1); -return x_7; +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_11 = lean_unsigned_to_nat(5u); +x_12 = l_Lean_Syntax_getArg(x_1, x_11); +x_13 = lean_unsigned_to_nat(0u); +x_14 = l_Lean_Syntax_getArg(x_12, x_13); +lean_dec(x_12); +x_15 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__1; +x_16 = l_Lean_Syntax_isToken(x_15, x_14); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; +lean_dec(x_14); +x_17 = lean_box(0); +x_18 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1(x_1, x_2, x_3, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_18; +} +else +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; lean_object* x_35; uint8_t x_36; lean_object* x_37; lean_object* x_38; +x_19 = l_Lean_Syntax_getArg(x_1, x_13); +lean_inc(x_19); +x_20 = l_Lean_Syntax_getKind(x_19); +x_21 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__3; +x_22 = lean_name_eq(x_20, x_21); +lean_dec(x_20); +x_23 = lean_ctor_get(x_8, 0); +x_24 = lean_ctor_get(x_8, 1); +x_25 = lean_ctor_get(x_8, 2); +x_26 = lean_ctor_get(x_8, 3); +x_27 = lean_ctor_get(x_8, 4); +x_28 = lean_ctor_get(x_8, 5); +x_29 = lean_ctor_get(x_8, 6); +x_30 = lean_ctor_get(x_8, 7); +x_31 = lean_ctor_get(x_8, 8); +x_32 = lean_ctor_get(x_8, 9); +x_33 = lean_ctor_get(x_8, 10); +x_34 = lean_ctor_get_uint8(x_8, sizeof(void*)*12); +x_35 = lean_ctor_get(x_8, 11); +x_36 = lean_ctor_get_uint8(x_8, sizeof(void*)*12 + 1); +x_37 = l_Lean_replaceRef(x_19, x_28); +lean_dec(x_19); +lean_inc(x_35); +lean_inc(x_33); +lean_inc(x_32); +lean_inc(x_31); +lean_inc(x_30); +lean_inc(x_29); +lean_inc(x_27); +lean_inc(x_26); +lean_inc(x_25); +lean_inc(x_24); +lean_inc(x_23); +x_38 = lean_alloc_ctor(0, 12, 2); +lean_ctor_set(x_38, 0, x_23); +lean_ctor_set(x_38, 1, x_24); +lean_ctor_set(x_38, 2, x_25); +lean_ctor_set(x_38, 3, x_26); +lean_ctor_set(x_38, 4, x_27); +lean_ctor_set(x_38, 5, x_37); +lean_ctor_set(x_38, 6, x_29); +lean_ctor_set(x_38, 7, x_30); +lean_ctor_set(x_38, 8, x_31); +lean_ctor_set(x_38, 9, x_32); +lean_ctor_set(x_38, 10, x_33); +lean_ctor_set(x_38, 11, x_35); +lean_ctor_set_uint8(x_38, sizeof(void*)*12, x_34); +lean_ctor_set_uint8(x_38, sizeof(void*)*12 + 1, x_36); +if (x_22 == 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; +x_39 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__13; +x_40 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__12; +x_41 = l_Lean_Linter_logLintIf___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__25(x_39, x_14, x_40, x_4, x_5, x_6, x_7, x_38, x_9, x_10); +lean_dec(x_14); +x_42 = lean_ctor_get(x_41, 0); +lean_inc(x_42); +x_43 = lean_ctor_get(x_41, 1); +lean_inc(x_43); +lean_dec(x_41); +x_44 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1(x_1, x_2, x_3, x_42, x_4, x_5, x_6, x_7, x_8, x_9, x_43); +lean_dec(x_42); +return x_44; +} +else +{ +lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_45 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__13; +x_46 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__20; +x_47 = l_Lean_Linter_logLintIf___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__25(x_45, x_14, x_46, x_4, x_5, x_6, x_7, x_38, x_9, x_10); +lean_dec(x_14); +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_Structure_0__Lean_Elab_Command_expandFields___lambda__1(x_1, x_2, x_3, x_48, x_4, x_5, x_6, x_7, x_8, x_9, x_49); +lean_dec(x_48); +return x_50; +} +} } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__5___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___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]; _start: { -lean_object* x_7; -x_7 = l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__5___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6); +uint8_t x_19; lean_object* x_20; +x_19 = lean_unbox(x_5); lean_dec(x_5); -return x_7; +x_20 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_19, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_11); +return x_20; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___boxed(lean_object** _args) { +lean_object* x_1 = _args[0]; +lean_object* x_2 = _args[1]; +lean_object* x_3 = _args[2]; +lean_object* x_4 = _args[3]; +lean_object* x_5 = _args[4]; +lean_object* x_6 = _args[5]; +lean_object* x_7 = _args[6]; +lean_object* x_8 = _args[7]; +lean_object* x_9 = _args[8]; +lean_object* x_10 = _args[9]; +lean_object* x_11 = _args[10]; +lean_object* x_12 = _args[11]; +lean_object* x_13 = _args[12]; +lean_object* x_14 = _args[13]; +lean_object* x_15 = _args[14]; +lean_object* x_16 = _args[15]; +lean_object* x_17 = _args[16]; _start: { -lean_object* x_9; -x_9 = l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +uint8_t x_18; size_t x_19; size_t x_20; lean_object* x_21; +x_18 = lean_unbox(x_2); +lean_dec(x_2); +x_19 = lean_unbox_usize(x_8); +lean_dec(x_8); +x_20 = lean_unbox_usize(x_9); +lean_dec(x_9); +x_21 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1(x_1, x_18, x_3, x_4, x_5, x_6, x_7, x_19, x_20, 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_7); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -return x_9; +return x_21; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___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_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__10(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__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); @@ -6430,707 +6664,631 @@ lean_dec(x_3); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___boxed(lean_object* x_1) { -_start: -{ -uint8_t x_2; lean_object* x_3; -x_2 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1(x_1); -lean_dec(x_1); -x_3 = lean_box(x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_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_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -uint8_t x_11; lean_object* x_12; -x_11 = lean_unbox(x_1); -lean_dec(x_1); -x_12 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___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_9); +lean_object* x_10; +x_10 = l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_8); -lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -return x_12; +lean_dec(x_4); +lean_dec(x_1); +return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; -x_9 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_7); +lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_1); return x_9; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, 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_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_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__11(x_1, x_12, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +uint8_t x_14; lean_object* x_15; +x_14 = lean_unbox(x_4); +lean_dec(x_4); +x_15 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__1(x_1, x_2, x_3, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_12); +lean_dec(x_11); lean_dec(x_10); +lean_dec(x_9); lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); lean_dec(x_1); -return x_14; +return x_15; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -lean_object* x_9; -x_9 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_7); -lean_dec(x_5); +uint8_t x_14; lean_object* x_15; +x_14 = lean_unbox(x_4); lean_dec(x_4); -lean_dec(x_3); +x_15 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2(x_1, x_2, x_3, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_6); lean_dec(x_1); -return x_9; +return x_15; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabDeclAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___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_9; -x_9 = l_Lean_Elab_elabDeclAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_7); -lean_dec(x_5); +uint8_t x_15; lean_object* x_16; +x_15 = lean_unbox(x_4); lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -return x_9; -} -} -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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) { -_start: -{ -lean_object* x_9; -x_9 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__13(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_16 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3(x_1, x_2, x_3, x_15, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); lean_dec(x_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_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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) { -_start: -{ -lean_object* x_10; -x_10 = l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__12(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_1); -return x_10; -} -} -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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) { -_start: -{ -lean_object* x_9; -x_9 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__16(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; +return x_16; } } -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_10; -x_10 = l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__15(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); +uint8_t x_13; lean_object* x_14; +x_13 = lean_unbox(x_5); lean_dec(x_5); +x_14 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4(x_1, x_2, x_3, x_4, x_13, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_4); lean_dec(x_1); -return x_10; +return x_14; } } -LEAN_EXPORT lean_object* l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_9; -x_9 = l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_7); +lean_object* x_13; +x_13 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___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); lean_dec(x_5); -lean_dec(x_4); lean_dec(x_3); -lean_dec(x_1); -return x_9; +return x_13; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -uint8_t x_14; uint8_t x_15; lean_object* x_16; -x_14 = lean_unbox(x_4); +size_t x_14; size_t x_15; lean_object* x_16; +x_14 = lean_unbox_usize(x_4); lean_dec(x_4); -x_15 = lean_unbox(x_5); +x_15 = lean_unbox_usize(x_5); lean_dec(x_5); -x_16 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__1(x_1, x_2, x_3, x_14, x_15, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_12); +x_16 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5(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_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_2); +lean_dec(x_3); lean_dec(x_1); return x_16; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___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: { -uint8_t x_14; uint8_t x_15; lean_object* x_16; -x_14 = lean_unbox(x_4); +size_t x_14; size_t x_15; lean_object* x_16; +x_14 = lean_unbox_usize(x_4); lean_dec(x_4); -x_15 = lean_unbox(x_6); -lean_dec(x_6); -x_16 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__2(x_1, x_2, x_3, x_14, x_5, x_15, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_12); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); +x_15 = lean_unbox_usize(x_5); lean_dec(x_5); -lean_dec(x_2); +x_16 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___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); lean_dec(x_1); return x_16; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -uint8_t x_14; lean_object* x_15; -x_14 = lean_unbox(x_3); -lean_dec(x_3); -x_15 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3(x_1, x_2, x_14, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_12); -lean_dec(x_10); +lean_object* x_12; +x_12 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___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_9); -lean_dec(x_8); -lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -return x_15; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; -x_9 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -return x_9; +return x_12; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_10; -x_10 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_object* x_11; +x_11 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, 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_2); lean_dec(x_1); -return x_10; +return x_11; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_structureSyntaxToView___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; -x_10 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_10 = lean_ctor_get(x_1, 2); +lean_inc(x_10); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); lean_dec(x_1); -return x_10; +x_12 = lean_box(0); +x_13 = l_Lean_Elab_addDeclarationRangesFromSyntax___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3(x_10, x_11, x_12, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_11); +return x_13; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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) { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_structureSyntaxToView___spec__1___closed__1() { _start: { -lean_object* x_10; -x_10 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -return x_10; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("', it is equal to structure constructor name", 44, 44); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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) { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_structureSyntaxToView___spec__1___closed__2() { _start: { -lean_object* x_9; -x_9 = l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17(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); -return x_9; +lean_object* x_1; lean_object* x_2; +x_1 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_structureSyntaxToView___spec__1___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__19___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_structureSyntaxToView___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: { -lean_object* x_9; -x_9 = l_Lean_Elab_getDeclarationRange___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__19(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -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_9; -} -} -LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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) { -_start: +uint8_t x_13; +x_13 = lean_usize_dec_eq(x_3, x_4); +if (x_13 == 0) { -lean_object* x_10; -x_10 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20(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_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -return x_10; +x_14 = lean_array_uget(x_2, x_3); +x_15 = lean_ctor_get(x_14, 2); +lean_inc(x_15); +x_16 = lean_ctor_get(x_1, 3); +x_17 = lean_name_eq(x_15, x_16); +lean_dec(x_15); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; size_t x_22; size_t x_23; +x_18 = lean_box(0); +lean_inc(x_10); +x_19 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_structureSyntaxToView___spec__1___lambda__1(x_14, x_18, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_19, 1); +lean_inc(x_21); +lean_dec(x_19); +x_22 = 1; +x_23 = lean_usize_add(x_3, x_22); +x_3 = x_23; +x_5 = x_20; +x_12 = x_21; +goto _start; } +else +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; +x_25 = lean_ctor_get(x_14, 0); +lean_inc(x_25); +x_26 = lean_ctor_get(x_14, 4); +lean_inc(x_26); +lean_dec(x_14); +x_27 = l_Lean_MessageData_ofName(x_26); +x_28 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___closed__2; +x_29 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_27); +x_30 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_structureSyntaxToView___spec__1___closed__2; +x_31 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_31, 0, x_29); +lean_ctor_set(x_31, 1, x_30); +x_32 = l_Lean_throwErrorAt___at___private_Lean_Elab_Binders_0__Lean_Elab_Term_elabBinderViews_loop___spec__1(x_25, x_31, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_25); +x_33 = !lean_is_exclusive(x_32); +if (x_33 == 0) +{ +return x_32; } -LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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) { -_start: +else { -lean_object* x_11; -x_11 = l_Lean_Elab_addAuxDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__18(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_9); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_11; +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_32, 0); +x_35 = lean_ctor_get(x_32, 1); +lean_inc(x_35); +lean_inc(x_34); +lean_dec(x_32); +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___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: +} +else { -lean_object* x_12; -x_12 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_object* x_37; lean_dec(x_10); -lean_dec(x_8); -lean_dec(x_7); lean_dec(x_6); -lean_dec(x_4); -lean_dec(x_1); -return x_12; +x_37 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_37, 0, x_5); +lean_ctor_set(x_37, 1, x_12); +return x_37; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_structureSyntaxToView___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_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18) { _start: { -lean_object* x_13; -x_13 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_11); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_1); -return x_13; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: +lean_object* x_19; +lean_inc(x_16); +lean_inc(x_12); +lean_inc(x_3); +x_19 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor(x_1, x_2, x_3, x_12, x_13, x_14, x_15, x_16, x_17, x_18); +if (lean_obj_tag(x_19) == 0) { -lean_object* x_11; -x_11 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_9); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_2); -lean_dec(x_1); -return x_11; -} -} -static lean_object* _init_l_Lean_Elab_Command_checkValidFieldModifier___lambda__1___closed__1() { -_start: +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_19, 1); +lean_inc(x_21); +lean_dec(x_19); +lean_inc(x_17); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_3); +x_22 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields(x_1, x_2, x_3, x_12, x_13, x_14, x_15, x_16, x_17, x_21); +if (lean_obj_tag(x_22) == 0) { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("invalid use of attributes in field declaration", 46, 46); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Command_checkValidFieldModifier___lambda__1___closed__2() { -_start: +uint8_t x_23; +x_23 = !lean_is_exclusive(x_22); +if (x_23 == 0) { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_checkValidFieldModifier___lambda__1___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; +x_24 = lean_ctor_get(x_22, 0); +x_25 = lean_ctor_get(x_22, 1); +x_26 = lean_array_get_size(x_24); +x_27 = lean_unsigned_to_nat(0u); +x_28 = lean_nat_dec_lt(x_27, x_26); +if (x_28 == 0) +{ +lean_object* x_29; +lean_dec(x_26); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +x_29 = lean_alloc_ctor(0, 12, 1); +lean_ctor_set(x_29, 0, x_1); +lean_ctor_set(x_29, 1, x_4); +lean_ctor_set(x_29, 2, x_2); +lean_ctor_set(x_29, 3, x_6); +lean_ctor_set(x_29, 4, x_3); +lean_ctor_set(x_29, 5, x_7); +lean_ctor_set(x_29, 6, x_8); +lean_ctor_set(x_29, 7, x_11); +lean_ctor_set(x_29, 8, x_9); +lean_ctor_set(x_29, 9, x_20); +lean_ctor_set(x_29, 10, x_24); +lean_ctor_set(x_29, 11, x_10); +lean_ctor_set_uint8(x_29, sizeof(void*)*12, x_5); +lean_ctor_set(x_22, 0, x_29); +return x_22; } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidFieldModifier___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_10 = lean_ctor_get(x_1, 1); -x_11 = lean_array_get_size(x_10); -x_12 = lean_unsigned_to_nat(0u); -x_13 = lean_nat_dec_eq(x_11, x_12); -lean_dec(x_11); -if (x_13 == 0) +uint8_t x_30; +x_30 = lean_nat_dec_le(x_26, x_26); +if (x_30 == 0) { -lean_object* x_14; lean_object* x_15; -x_14 = l_Lean_Elab_Command_checkValidFieldModifier___lambda__1___closed__2; -x_15 = l_Lean_throwError___at_Lean_Elab_Term_throwErrorIfErrors___spec__1(x_14, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_15; +lean_object* x_31; +lean_dec(x_26); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +x_31 = lean_alloc_ctor(0, 12, 1); +lean_ctor_set(x_31, 0, x_1); +lean_ctor_set(x_31, 1, x_4); +lean_ctor_set(x_31, 2, x_2); +lean_ctor_set(x_31, 3, x_6); +lean_ctor_set(x_31, 4, x_3); +lean_ctor_set(x_31, 5, x_7); +lean_ctor_set(x_31, 6, x_8); +lean_ctor_set(x_31, 7, x_11); +lean_ctor_set(x_31, 8, x_9); +lean_ctor_set(x_31, 9, x_20); +lean_ctor_set(x_31, 10, x_24); +lean_ctor_set(x_31, 11, x_10); +lean_ctor_set_uint8(x_31, sizeof(void*)*12, x_5); +lean_ctor_set(x_22, 0, x_31); +return x_22; } else { -lean_object* x_16; lean_object* x_17; -lean_dec(x_3); -x_16 = lean_box(0); -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_16); -lean_ctor_set(x_17, 1, x_9); -return x_17; -} -} -} -static lean_object* _init_l_Lean_Elab_Command_checkValidFieldModifier___lambda__2___closed__1() { -_start: +size_t x_32; size_t x_33; lean_object* x_34; lean_object* x_35; +lean_free_object(x_22); +x_32 = 0; +x_33 = lean_usize_of_nat(x_26); +lean_dec(x_26); +x_34 = lean_box(0); +x_35 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_structureSyntaxToView___spec__1(x_20, x_24, x_32, x_33, x_34, x_12, x_13, x_14, x_15, x_16, x_17, x_25); +lean_dec(x_17); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +if (lean_obj_tag(x_35) == 0) { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("invalid use of 'unsafe' in field declaration", 44, 44); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Command_checkValidFieldModifier___lambda__2___closed__2() { -_start: +uint8_t x_36; +x_36 = !lean_is_exclusive(x_35); +if (x_36 == 0) { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_checkValidFieldModifier___lambda__2___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} +lean_object* x_37; lean_object* x_38; +x_37 = lean_ctor_get(x_35, 0); +lean_dec(x_37); +x_38 = lean_alloc_ctor(0, 12, 1); +lean_ctor_set(x_38, 0, x_1); +lean_ctor_set(x_38, 1, x_4); +lean_ctor_set(x_38, 2, x_2); +lean_ctor_set(x_38, 3, x_6); +lean_ctor_set(x_38, 4, x_3); +lean_ctor_set(x_38, 5, x_7); +lean_ctor_set(x_38, 6, x_8); +lean_ctor_set(x_38, 7, x_11); +lean_ctor_set(x_38, 8, x_9); +lean_ctor_set(x_38, 9, x_20); +lean_ctor_set(x_38, 10, x_24); +lean_ctor_set(x_38, 11, x_10); +lean_ctor_set_uint8(x_38, sizeof(void*)*12, x_5); +lean_ctor_set(x_35, 0, x_38); +return x_35; } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidFieldModifier___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -uint8_t x_10; -x_10 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 3); -if (x_10 == 0) +else { -lean_object* x_11; lean_object* x_12; -x_11 = lean_box(0); -x_12 = l_Lean_Elab_Command_checkValidFieldModifier___lambda__1(x_1, x_11, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_12; +lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = lean_ctor_get(x_35, 1); +lean_inc(x_39); +lean_dec(x_35); +x_40 = lean_alloc_ctor(0, 12, 1); +lean_ctor_set(x_40, 0, x_1); +lean_ctor_set(x_40, 1, x_4); +lean_ctor_set(x_40, 2, x_2); +lean_ctor_set(x_40, 3, x_6); +lean_ctor_set(x_40, 4, x_3); +lean_ctor_set(x_40, 5, x_7); +lean_ctor_set(x_40, 6, x_8); +lean_ctor_set(x_40, 7, x_11); +lean_ctor_set(x_40, 8, x_9); +lean_ctor_set(x_40, 9, x_20); +lean_ctor_set(x_40, 10, x_24); +lean_ctor_set(x_40, 11, x_10); +lean_ctor_set_uint8(x_40, sizeof(void*)*12, x_5); +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; +} } else { -lean_object* x_13; lean_object* x_14; uint8_t x_15; -x_13 = l_Lean_Elab_Command_checkValidFieldModifier___lambda__2___closed__2; -x_14 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -x_15 = !lean_is_exclusive(x_14); -if (x_15 == 0) +uint8_t x_42; +lean_dec(x_24); +lean_dec(x_20); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_42 = !lean_is_exclusive(x_35); +if (x_42 == 0) { -return x_14; +return x_35; } else { -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_14, 0); -x_17 = lean_ctor_get(x_14, 1); -lean_inc(x_17); -lean_inc(x_16); -lean_dec(x_14); -x_18 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_18, 0, x_16); -lean_ctor_set(x_18, 1, x_17); -return x_18; -} -} -} +lean_object* x_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; } -static lean_object* _init_l_Lean_Elab_Command_checkValidFieldModifier___lambda__3___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("invalid use of 'partial' in field declaration", 45, 45); -return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_checkValidFieldModifier___lambda__3___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_checkValidFieldModifier___lambda__3___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidFieldModifier___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: +else { -uint8_t x_10; -x_10 = l_Lean_Elab_Modifiers_isPartial(x_1); -if (x_10 == 0) +lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; uint8_t x_50; +x_46 = lean_ctor_get(x_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_array_get_size(x_46); +x_49 = lean_unsigned_to_nat(0u); +x_50 = lean_nat_dec_lt(x_49, x_48); +if (x_50 == 0) { -lean_object* x_11; lean_object* x_12; -x_11 = lean_box(0); -x_12 = l_Lean_Elab_Command_checkValidFieldModifier___lambda__2(x_1, x_11, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_12; +lean_object* x_51; lean_object* x_52; +lean_dec(x_48); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +x_51 = lean_alloc_ctor(0, 12, 1); +lean_ctor_set(x_51, 0, x_1); +lean_ctor_set(x_51, 1, x_4); +lean_ctor_set(x_51, 2, x_2); +lean_ctor_set(x_51, 3, x_6); +lean_ctor_set(x_51, 4, x_3); +lean_ctor_set(x_51, 5, x_7); +lean_ctor_set(x_51, 6, x_8); +lean_ctor_set(x_51, 7, x_11); +lean_ctor_set(x_51, 8, x_9); +lean_ctor_set(x_51, 9, x_20); +lean_ctor_set(x_51, 10, x_46); +lean_ctor_set(x_51, 11, x_10); +lean_ctor_set_uint8(x_51, sizeof(void*)*12, x_5); +x_52 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_52, 0, x_51); +lean_ctor_set(x_52, 1, x_47); +return x_52; } else { -lean_object* x_13; lean_object* x_14; uint8_t x_15; -x_13 = l_Lean_Elab_Command_checkValidFieldModifier___lambda__3___closed__2; -x_14 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -x_15 = !lean_is_exclusive(x_14); -if (x_15 == 0) +uint8_t x_53; +x_53 = lean_nat_dec_le(x_48, x_48); +if (x_53 == 0) { -return x_14; +lean_object* x_54; lean_object* x_55; +lean_dec(x_48); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +x_54 = lean_alloc_ctor(0, 12, 1); +lean_ctor_set(x_54, 0, x_1); +lean_ctor_set(x_54, 1, x_4); +lean_ctor_set(x_54, 2, x_2); +lean_ctor_set(x_54, 3, x_6); +lean_ctor_set(x_54, 4, x_3); +lean_ctor_set(x_54, 5, x_7); +lean_ctor_set(x_54, 6, x_8); +lean_ctor_set(x_54, 7, x_11); +lean_ctor_set(x_54, 8, x_9); +lean_ctor_set(x_54, 9, x_20); +lean_ctor_set(x_54, 10, x_46); +lean_ctor_set(x_54, 11, x_10); +lean_ctor_set_uint8(x_54, sizeof(void*)*12, x_5); +x_55 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_55, 0, x_54); +lean_ctor_set(x_55, 1, x_47); +return x_55; } else { -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_14, 0); -x_17 = lean_ctor_get(x_14, 1); -lean_inc(x_17); -lean_inc(x_16); -lean_dec(x_14); -x_18 = lean_alloc_ctor(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_Elab_Command_checkValidFieldModifier___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("invalid use of 'noncomputable' in field declaration", 51, 51); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Command_checkValidFieldModifier___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_checkValidFieldModifier___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidFieldModifier(lean_object* x_1, lean_object* x_2, lean_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_ctor_get_uint8(x_1, sizeof(void*)*2 + 1); -if (x_9 == 0) -{ -lean_object* x_10; lean_object* x_11; -x_10 = lean_box(0); -x_11 = l_Lean_Elab_Command_checkValidFieldModifier___lambda__3(x_1, x_10, 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; uint8_t x_14; -x_12 = l_Lean_Elab_Command_checkValidFieldModifier___closed__2; -x_13 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -x_14 = !lean_is_exclusive(x_13); -if (x_14 == 0) -{ -return x_13; -} -else -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = lean_ctor_get(x_13, 0); -x_16 = lean_ctor_get(x_13, 1); -lean_inc(x_16); -lean_inc(x_15); +size_t x_56; size_t x_57; lean_object* x_58; lean_object* x_59; +x_56 = 0; +x_57 = lean_usize_of_nat(x_48); +lean_dec(x_48); +x_58 = lean_box(0); +x_59 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_structureSyntaxToView___spec__1(x_20, x_46, x_56, x_57, x_58, x_12, x_13, x_14, x_15, x_16, x_17, x_47); +lean_dec(x_17); +lean_dec(x_15); +lean_dec(x_14); lean_dec(x_13); -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_Command_checkValidFieldModifier___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +if (lean_obj_tag(x_59) == 0) { -lean_object* x_10; -x_10 = l_Lean_Elab_Command_checkValidFieldModifier___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -return x_10; -} +lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; +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; +} else { + lean_dec_ref(x_59); + x_61 = lean_box(0); } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidFieldModifier___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; -x_10 = l_Lean_Elab_Command_checkValidFieldModifier___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -return x_10; +x_62 = lean_alloc_ctor(0, 12, 1); +lean_ctor_set(x_62, 0, x_1); +lean_ctor_set(x_62, 1, x_4); +lean_ctor_set(x_62, 2, x_2); +lean_ctor_set(x_62, 3, x_6); +lean_ctor_set(x_62, 4, x_3); +lean_ctor_set(x_62, 5, x_7); +lean_ctor_set(x_62, 6, x_8); +lean_ctor_set(x_62, 7, x_11); +lean_ctor_set(x_62, 8, x_9); +lean_ctor_set(x_62, 9, x_20); +lean_ctor_set(x_62, 10, x_46); +lean_ctor_set(x_62, 11, x_10); +lean_ctor_set_uint8(x_62, sizeof(void*)*12, x_5); +if (lean_is_scalar(x_61)) { + x_63 = lean_alloc_ctor(0, 2, 0); +} else { + x_63 = x_61; } +lean_ctor_set(x_63, 0, x_62); +lean_ctor_set(x_63, 1, x_60); +return x_63; } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidFieldModifier___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +else { -lean_object* x_10; -x_10 = l_Lean_Elab_Command_checkValidFieldModifier___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; +lean_dec(x_46); +lean_dec(x_20); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -return x_10; +x_64 = lean_ctor_get(x_59, 0); +lean_inc(x_64); +x_65 = lean_ctor_get(x_59, 1); +lean_inc(x_65); +if (lean_is_exclusive(x_59)) { + lean_ctor_release(x_59, 0); + lean_ctor_release(x_59, 1); + x_66 = x_59; +} else { + lean_dec_ref(x_59); + x_66 = lean_box(0); } +if (lean_is_scalar(x_66)) { + x_67 = lean_alloc_ctor(1, 2, 0); +} else { + x_67 = x_66; } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidFieldModifier___boxed(lean_object* x_1, lean_object* x_2, lean_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_Command_checkValidFieldModifier(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); -return x_9; +lean_ctor_set(x_67, 0, x_64); +lean_ctor_set(x_67, 1, x_65); +return x_67; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___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_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18) { -_start: -{ -lean_object* x_19; uint8_t x_20; lean_object* x_21; -lean_inc(x_2); -x_19 = l_Lean_Name_append(x_1, x_2); -x_20 = lean_ctor_get_uint8(x_3, sizeof(void*)*2); -lean_inc(x_12); -x_21 = l_Lean_Elab_applyVisibility___at_Lean_Elab_Term_expandDeclId___spec__5(x_20, x_19, x_12, x_13, x_14, x_15, x_16, x_17, x_18); -if (lean_obj_tag(x_21) == 0) -{ -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_ctor_get(x_3, 0); -lean_inc(x_24); -lean_inc(x_22); -x_25 = l_Lean_addDocString_x27___at_Lean_Elab_Term_expandDeclId___spec__8(x_22, x_24, x_12, x_13, x_14, x_15, x_16, x_17, x_23); -if (lean_obj_tag(x_25) == 0) -{ -uint8_t x_26; -x_26 = !lean_is_exclusive(x_25); -if (x_26 == 0) -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_25, 0); -lean_dec(x_27); -x_28 = lean_alloc_ctor(0, 8, 1); -lean_ctor_set(x_28, 0, x_4); -lean_ctor_set(x_28, 1, x_3); -lean_ctor_set(x_28, 2, x_22); -lean_ctor_set(x_28, 3, x_2); -lean_ctor_set(x_28, 4, x_6); -lean_ctor_set(x_28, 5, x_7); -lean_ctor_set(x_28, 6, x_8); -lean_ctor_set(x_28, 7, x_9); -lean_ctor_set_uint8(x_28, sizeof(void*)*8, x_5); -x_29 = lean_array_push(x_10, x_28); -lean_ctor_set(x_25, 0, x_29); -return x_25; } -else -{ -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_30 = lean_ctor_get(x_25, 1); -lean_inc(x_30); -lean_dec(x_25); -x_31 = lean_alloc_ctor(0, 8, 1); -lean_ctor_set(x_31, 0, x_4); -lean_ctor_set(x_31, 1, x_3); -lean_ctor_set(x_31, 2, x_22); -lean_ctor_set(x_31, 3, x_2); -lean_ctor_set(x_31, 4, x_6); -lean_ctor_set(x_31, 5, x_7); -lean_ctor_set(x_31, 6, x_8); -lean_ctor_set(x_31, 7, x_9); -lean_ctor_set_uint8(x_31, sizeof(void*)*8, x_5); -x_32 = lean_array_push(x_10, x_31); -x_33 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_33, 0, x_32); -lean_ctor_set(x_33, 1, x_30); -return x_33; } } else { -uint8_t x_34; -lean_dec(x_22); +uint8_t x_68; +lean_dec(x_20); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -7139,30 +7297,37 @@ lean_dec(x_6); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_34 = !lean_is_exclusive(x_25); -if (x_34 == 0) +lean_dec(x_1); +x_68 = !lean_is_exclusive(x_22); +if (x_68 == 0) { -return x_25; +return x_22; } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_35 = lean_ctor_get(x_25, 0); -x_36 = lean_ctor_get(x_25, 1); -lean_inc(x_36); -lean_inc(x_35); -lean_dec(x_25); -x_37 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -return x_37; +lean_object* x_69; lean_object* x_70; lean_object* x_71; +x_69 = lean_ctor_get(x_22, 0); +x_70 = lean_ctor_get(x_22, 1); +lean_inc(x_70); +lean_inc(x_69); +lean_dec(x_22); +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_38; +uint8_t x_72; +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); @@ -7171,1729 +7336,1257 @@ lean_dec(x_6); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_38 = !lean_is_exclusive(x_21); -if (x_38 == 0) +lean_dec(x_1); +x_72 = !lean_is_exclusive(x_19); +if (x_72 == 0) { -return x_21; +return x_19; } else { -lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_39 = lean_ctor_get(x_21, 0); -x_40 = lean_ctor_get(x_21, 1); -lean_inc(x_40); -lean_inc(x_39); -lean_dec(x_21); -x_41 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_41, 0, x_39); -lean_ctor_set(x_41, 1, x_40); -return x_41; -} -} -} -} -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___closed__1() { -_start: +lean_object* x_73; lean_object* x_74; lean_object* x_75; +x_73 = lean_ctor_get(x_19, 0); +x_74 = lean_ctor_get(x_19, 1); +lean_inc(x_74); +lean_inc(x_73); +lean_dec(x_19); +x_75 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_75, 0, x_73); +lean_ctor_set(x_75, 1, x_74); +return x_75; +} +} +} +} +static lean_object* _init_l_Lean_Elab_Command_structureSyntaxToView___closed__1() { +_start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("invalid field name '", 20, 20); +x_1 = lean_mk_string_unchecked("sort", 4, 4); return x_1; } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___closed__2() { +static lean_object* _init_l_Lean_Elab_Command_structureSyntaxToView___closed__2() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__6; +x_2 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__1; +x_3 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__2; +x_4 = l_Lean_Elab_Command_structureSyntaxToView___closed__1; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___closed__3() { +static lean_object* _init_l_Lean_Elab_Command_structureSyntaxToView___closed__3() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("', field names must be atomic", 29, 29); +x_1 = lean_mk_string_unchecked("Sort", 4, 4); return x_1; } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___closed__4() { +static lean_object* _init_l_Lean_Elab_Command_structureSyntaxToView___closed__4() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___closed__3; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Level", 5, 5); +return x_1; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___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, size_t x_8, size_t x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { +static lean_object* _init_l_Lean_Elab_Command_structureSyntaxToView___closed__5() { _start: { -uint8_t x_18; -x_18 = lean_usize_dec_eq(x_8, x_9); -if (x_18 == 0) +lean_object* x_1; +x_1 = lean_mk_string_unchecked("hole", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Command_structureSyntaxToView___closed__6() { +_start: { -lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; lean_object* x_35; uint8_t x_36; lean_object* x_37; lean_object* x_38; -x_19 = lean_array_uget(x_7, x_8); -x_20 = l_Lean_Syntax_getId(x_19); -lean_inc(x_20); -x_21 = lean_erase_macro_scopes(x_20); -x_22 = l_Lean_Name_isAtomic(x_21); -x_23 = lean_ctor_get(x_15, 0); -x_24 = lean_ctor_get(x_15, 1); -x_25 = lean_ctor_get(x_15, 2); -x_26 = lean_ctor_get(x_15, 3); -x_27 = lean_ctor_get(x_15, 4); -x_28 = lean_ctor_get(x_15, 5); -x_29 = lean_ctor_get(x_15, 6); -x_30 = lean_ctor_get(x_15, 7); -x_31 = lean_ctor_get(x_15, 8); -x_32 = lean_ctor_get(x_15, 9); -x_33 = lean_ctor_get(x_15, 10); -x_34 = lean_ctor_get_uint8(x_15, sizeof(void*)*12); -x_35 = lean_ctor_get(x_15, 11); -x_36 = lean_ctor_get_uint8(x_15, sizeof(void*)*12 + 1); -x_37 = l_Lean_replaceRef(x_19, x_28); -lean_inc(x_35); -lean_inc(x_33); -lean_inc(x_32); -lean_inc(x_31); -lean_inc(x_30); -lean_inc(x_29); -lean_inc(x_27); -lean_inc(x_26); -lean_inc(x_25); -lean_inc(x_24); -lean_inc(x_23); -x_38 = lean_alloc_ctor(0, 12, 2); -lean_ctor_set(x_38, 0, x_23); -lean_ctor_set(x_38, 1, x_24); -lean_ctor_set(x_38, 2, x_25); -lean_ctor_set(x_38, 3, x_26); -lean_ctor_set(x_38, 4, x_27); -lean_ctor_set(x_38, 5, x_37); -lean_ctor_set(x_38, 6, x_29); -lean_ctor_set(x_38, 7, x_30); -lean_ctor_set(x_38, 8, x_31); -lean_ctor_set(x_38, 9, x_32); -lean_ctor_set(x_38, 10, x_33); -lean_ctor_set(x_38, 11, x_35); -lean_ctor_set_uint8(x_38, sizeof(void*)*12, x_34); -lean_ctor_set_uint8(x_38, sizeof(void*)*12 + 1, x_36); -if (x_22 == 0) +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__6; +x_2 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__1; +x_3 = l_Lean_Elab_Command_structureSyntaxToView___closed__4; +x_4 = l_Lean_Elab_Command_structureSyntaxToView___closed__5; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Elab_Command_structureSyntaxToView___closed__7() { +_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_object* x_45; uint8_t x_46; -lean_dec(x_20); -lean_dec(x_10); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_39 = lean_erase_macro_scopes(x_21); -x_40 = l_Lean_MessageData_ofName(x_39); -x_41 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___closed__2; -x_42 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_42, 0, x_41); -lean_ctor_set(x_42, 1, x_40); -x_43 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___closed__4; -x_44 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_44, 0, x_42); -lean_ctor_set(x_44, 1, x_43); -x_45 = l_Lean_throwErrorAt___at___private_Lean_Elab_Binders_0__Lean_Elab_Term_elabBinderViews_loop___spec__1(x_19, x_44, x_11, x_12, x_13, x_14, x_38, x_16, x_17); -lean_dec(x_19); -x_46 = !lean_is_exclusive(x_45); -if (x_46 == 0) +lean_object* x_1; +x_1 = lean_mk_string_unchecked("_", 1, 1); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Command_structureSyntaxToView___closed__8() { +_start: { -return x_45; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__14; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } -else +} +static lean_object* _init_l_Lean_Elab_Command_structureSyntaxToView___closed__9() { +_start: { -lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_47 = lean_ctor_get(x_45, 0); -x_48 = lean_ctor_get(x_45, 1); -lean_inc(x_48); -lean_inc(x_47); -lean_dec(x_45); -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; +uint8_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = 0; +x_2 = l_Lean_Elab_Command_structureSyntaxToView___closed__8; +x_3 = lean_box(0); +x_4 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_4, 0, x_2); +lean_ctor_set(x_4, 1, x_3); +lean_ctor_set_uint8(x_4, sizeof(void*)*2, x_1); +return x_4; } } -else +LEAN_EXPORT lean_object* l_Lean_Elab_Command_structureSyntaxToView(lean_object* x_1, lean_object* x_2, lean_object* x_3, 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_50; lean_object* x_51; -x_50 = lean_box(0); +lean_object* x_10; +lean_inc(x_3); +x_10 = l_Lean_Elab_Command_checkValidInductiveModifier___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_10) == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_11 = lean_ctor_get(x_10, 1); lean_inc(x_11); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); +lean_dec(x_10); +x_12 = lean_unsigned_to_nat(0u); +x_13 = l_Lean_Syntax_getArg(x_2, x_12); +x_14 = l_Lean_Syntax_getKind(x_13); +x_15 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__3; +x_16 = lean_name_eq(x_14, x_15); +lean_dec(x_14); +x_17 = lean_unsigned_to_nat(1u); +x_18 = l_Lean_Syntax_getArg(x_2, x_17); +x_19 = lean_ctor_get(x_7, 6); +lean_inc(x_19); +x_20 = l_Lean_Elab_Term_getLevelNames___rarg(x_4, x_5, x_6, x_7, x_8, x_11); +if (x_16 == 0) +{ +lean_object* x_102; lean_object* x_103; +x_102 = lean_ctor_get(x_20, 0); +lean_inc(x_102); +x_103 = lean_ctor_get(x_20, 1); +lean_inc(x_103); +lean_dec(x_20); +x_21 = x_1; +x_22 = x_102; +x_23 = x_103; +goto block_101; +} +else +{ +lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; +x_104 = lean_ctor_get(x_20, 0); +lean_inc(x_104); +x_105 = lean_ctor_get(x_20, 1); +lean_inc(x_105); +lean_dec(x_20); +x_106 = l_Lean_Elab_Command_structureSyntaxToView___closed__9; +x_107 = l_Lean_Elab_Modifiers_addAttr(x_1, x_106); +x_21 = x_107; +x_22 = x_104; +x_23 = x_105; +goto block_101; +} +block_101: +{ +lean_object* x_24; +lean_inc(x_7); lean_inc(x_3); -lean_inc(x_1); -x_51 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___lambda__1(x_1, x_21, x_3, x_19, x_2, x_20, x_4, x_5, x_6, x_10, x_50, x_11, x_12, x_13, x_14, x_38, x_16, x_17); -lean_dec(x_38); -if (lean_obj_tag(x_51) == 0) +lean_inc(x_21); +x_24 = l_Lean_Elab_Term_expandDeclId(x_19, x_22, x_18, x_21, x_3, x_4, x_5, x_6, x_7, x_8, x_23); +if (lean_obj_tag(x_24) == 0) { -lean_object* x_52; lean_object* x_53; size_t x_54; size_t x_55; -x_52 = lean_ctor_get(x_51, 0); -lean_inc(x_52); -x_53 = lean_ctor_get(x_51, 1); -lean_inc(x_53); -lean_dec(x_51); -x_54 = 1; -x_55 = lean_usize_add(x_8, x_54); -x_8 = x_55; -x_10 = x_52; -x_17 = x_53; -goto _start; +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; uint8_t x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; +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); +x_28 = lean_ctor_get(x_25, 1); +lean_inc(x_28); +x_29 = lean_ctor_get(x_25, 2); +lean_inc(x_29); +lean_dec(x_25); +x_30 = lean_ctor_get(x_21, 0); +lean_inc(x_30); +lean_inc(x_7); +lean_inc(x_2); +lean_inc(x_28); +x_31 = l_Lean_Elab_addDeclarationRangesForBuiltin___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2(x_28, x_30, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_26); +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; +} else { + lean_dec_ref(x_31); + x_33 = lean_box(0); +} +x_34 = lean_unsigned_to_nat(2u); +x_35 = l_Lean_Syntax_getArg(x_2, x_34); +x_36 = lean_unsigned_to_nat(3u); +x_37 = l_Lean_Syntax_getArg(x_2, x_36); +x_38 = l_Lean_Syntax_isNone(x_37); +x_39 = lean_unsigned_to_nat(4u); +x_40 = l_Lean_Syntax_getArg(x_2, x_39); +x_41 = lean_unsigned_to_nat(6u); +x_42 = l_Lean_Syntax_getArg(x_2, x_41); +lean_inc(x_8); +lean_inc(x_7); +x_43 = l_Lean_Elab_getOptDerivingClasses(x_42, x_7, x_8, x_32); +if (x_38 == 0) +{ +if (lean_obj_tag(x_43) == 0) +{ +lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; +x_81 = lean_ctor_get(x_43, 0); +lean_inc(x_81); +x_82 = lean_ctor_get(x_43, 1); +lean_inc(x_82); +lean_dec(x_43); +x_83 = l_Lean_Syntax_getArg(x_37, x_12); +lean_dec(x_37); +x_84 = l_Lean_Syntax_getArg(x_83, x_17); +lean_dec(x_83); +x_85 = l_Lean_Syntax_getSepArgs(x_84); +lean_dec(x_84); +x_44 = x_85; +x_45 = x_81; +x_46 = x_82; +goto block_80; } else { -uint8_t x_57; -lean_dec(x_11); +uint8_t x_86; +lean_dec(x_40); +lean_dec(x_37); +lean_dec(x_35); +lean_dec(x_33); +lean_dec(x_29); +lean_dec(x_28); +lean_dec(x_27); +lean_dec(x_21); +lean_dec(x_18); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_1); -x_57 = !lean_is_exclusive(x_51); -if (x_57 == 0) +lean_dec(x_2); +x_86 = !lean_is_exclusive(x_43); +if (x_86 == 0) { -return x_51; +return x_43; } else { -lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_58 = lean_ctor_get(x_51, 0); -x_59 = lean_ctor_get(x_51, 1); -lean_inc(x_59); -lean_inc(x_58); -lean_dec(x_51); -x_60 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_60, 0, x_58); -lean_ctor_set(x_60, 1, x_59); -return x_60; +lean_object* x_87; lean_object* x_88; lean_object* x_89; +x_87 = lean_ctor_get(x_43, 0); +x_88 = lean_ctor_get(x_43, 1); +lean_inc(x_88); +lean_inc(x_87); +lean_dec(x_43); +x_89 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_89, 0, x_87); +lean_ctor_set(x_89, 1, x_88); +return x_89; } } } +else +{ +lean_dec(x_37); +if (lean_obj_tag(x_43) == 0) +{ +lean_object* x_90; lean_object* x_91; lean_object* x_92; +x_90 = lean_ctor_get(x_43, 0); +lean_inc(x_90); +x_91 = lean_ctor_get(x_43, 1); +lean_inc(x_91); +lean_dec(x_43); +x_92 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__1; +x_44 = x_92; +x_45 = x_90; +x_46 = x_91; +goto block_80; } else { -lean_object* x_61; -lean_dec(x_11); +uint8_t x_93; +lean_dec(x_40); +lean_dec(x_35); +lean_dec(x_33); +lean_dec(x_29); +lean_dec(x_28); +lean_dec(x_27); +lean_dec(x_21); +lean_dec(x_18); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_1); -x_61 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_61, 0, x_10); -lean_ctor_set(x_61, 1, x_17); -return x_61; +lean_dec(x_2); +x_93 = !lean_is_exclusive(x_43); +if (x_93 == 0) +{ +return x_43; } +else +{ +lean_object* x_94; lean_object* x_95; lean_object* x_96; +x_94 = lean_ctor_get(x_43, 0); +x_95 = lean_ctor_get(x_43, 1); +lean_inc(x_95); +lean_inc(x_94); +lean_dec(x_43); +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; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___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; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; -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_is_exclusive(x_12); -if (x_13 == 0) +} +block_80: { -lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; -x_14 = lean_ctor_get(x_12, 0); -x_15 = lean_ctor_get(x_12, 1); -x_16 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(x_14, x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_15); -lean_dec(x_2); -x_17 = !lean_is_exclusive(x_16); -if (x_17 == 0) +uint8_t x_47; +x_47 = l_Lean_Syntax_isNone(x_40); +if (x_47 == 0) { -lean_object* x_18; -x_18 = lean_ctor_get(x_16, 0); -lean_ctor_set(x_12, 1, x_18); -lean_ctor_set(x_12, 0, x_11); -lean_ctor_set_tag(x_16, 1); -lean_ctor_set(x_16, 0, x_12); -return x_16; +lean_object* x_48; lean_object* x_49; lean_object* x_50; +lean_dec(x_33); +x_48 = l_Lean_Syntax_getArg(x_40, x_12); +lean_dec(x_40); +x_49 = l_Lean_Syntax_getArg(x_48, x_17); +lean_dec(x_48); +x_50 = l_Lean_Elab_Command_structureSyntaxToView___lambda__1(x_2, x_21, x_28, x_18, x_16, x_27, x_29, x_35, x_44, x_45, x_49, x_3, x_4, x_5, x_6, x_7, x_8, x_46); +return x_50; } 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_12, 1, x_19); -lean_ctor_set(x_12, 0, x_11); -x_21 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_21, 0, x_12); -lean_ctor_set(x_21, 1, x_20); -return x_21; +lean_object* x_51; uint8_t x_52; lean_object* x_53; lean_object* x_54; uint8_t x_55; +lean_dec(x_40); +x_51 = lean_ctor_get(x_7, 5); +lean_inc(x_51); +x_52 = 0; +x_53 = l_Lean_SourceInfo_fromRef(x_51, x_52); +lean_dec(x_51); +x_54 = lean_st_ref_get(x_8, x_46); +x_55 = !lean_is_exclusive(x_54); +if (x_55 == 0) +{ +lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; 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_56 = lean_ctor_get(x_54, 1); +x_57 = lean_ctor_get(x_54, 0); +lean_dec(x_57); +x_58 = l_Lean_Elab_Command_structureSyntaxToView___closed__3; +lean_inc(x_53); +lean_ctor_set_tag(x_54, 2); +lean_ctor_set(x_54, 1, x_58); +lean_ctor_set(x_54, 0, x_53); +x_59 = l_Lean_Elab_Command_structureSyntaxToView___closed__7; +lean_inc(x_53); +if (lean_is_scalar(x_33)) { + x_60 = lean_alloc_ctor(2, 2, 0); +} else { + x_60 = x_33; + lean_ctor_set_tag(x_60, 2); } +lean_ctor_set(x_60, 0, x_53); +lean_ctor_set(x_60, 1, x_59); +x_61 = l_Lean_Elab_Command_structureSyntaxToView___closed__6; +lean_inc(x_53); +x_62 = l_Lean_Syntax_node1(x_53, x_61, x_60); +x_63 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__10; +lean_inc(x_53); +x_64 = l_Lean_Syntax_node1(x_53, x_63, x_62); +x_65 = l_Lean_Elab_Command_structureSyntaxToView___closed__2; +x_66 = l_Lean_Syntax_node2(x_53, x_65, x_54, x_64); +x_67 = l_Lean_Elab_Command_structureSyntaxToView___lambda__1(x_2, x_21, x_28, x_18, x_16, x_27, x_29, x_35, x_44, x_45, x_66, x_3, x_4, x_5, x_6, x_7, x_8, x_56); +return x_67; } 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; -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 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(x_22, x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_23); -lean_dec(x_2); -x_25 = lean_ctor_get(x_24, 0); -lean_inc(x_25); -x_26 = lean_ctor_get(x_24, 1); -lean_inc(x_26); -if (lean_is_exclusive(x_24)) { - lean_ctor_release(x_24, 0); - lean_ctor_release(x_24, 1); - x_27 = x_24; +lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; +x_68 = lean_ctor_get(x_54, 1); +lean_inc(x_68); +lean_dec(x_54); +x_69 = l_Lean_Elab_Command_structureSyntaxToView___closed__3; +lean_inc(x_53); +x_70 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_70, 0, x_53); +lean_ctor_set(x_70, 1, x_69); +x_71 = l_Lean_Elab_Command_structureSyntaxToView___closed__7; +lean_inc(x_53); +if (lean_is_scalar(x_33)) { + x_72 = lean_alloc_ctor(2, 2, 0); } else { - lean_dec_ref(x_24); - x_27 = lean_box(0); + x_72 = x_33; + lean_ctor_set_tag(x_72, 2); } -x_28 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_28, 0, x_11); -lean_ctor_set(x_28, 1, x_25); -if (lean_is_scalar(x_27)) { - x_29 = lean_alloc_ctor(1, 2, 0); -} else { - x_29 = x_27; - lean_ctor_set_tag(x_29, 1); +lean_ctor_set(x_72, 0, x_53); +lean_ctor_set(x_72, 1, x_71); +x_73 = l_Lean_Elab_Command_structureSyntaxToView___closed__6; +lean_inc(x_53); +x_74 = l_Lean_Syntax_node1(x_53, x_73, x_72); +x_75 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__10; +lean_inc(x_53); +x_76 = l_Lean_Syntax_node1(x_53, x_75, x_74); +x_77 = l_Lean_Elab_Command_structureSyntaxToView___closed__2; +x_78 = l_Lean_Syntax_node2(x_53, x_77, x_70, x_76); +x_79 = l_Lean_Elab_Command_structureSyntaxToView___lambda__1(x_2, x_21, x_28, x_18, x_16, x_27, x_29, x_35, x_44, x_45, x_78, x_3, x_4, x_5, x_6, x_7, x_8, x_68); +return x_79; } -lean_ctor_set(x_29, 0, x_28); -lean_ctor_set(x_29, 1, x_26); -return x_29; } } } -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -uint8_t x_10; -x_10 = !lean_is_exclusive(x_7); -if (x_10 == 0) +else { -lean_object* x_11; lean_object* x_12; lean_object* x_13; -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_Structure_0__Lean_Elab_Command_expandFields___spec__3(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +uint8_t x_97; +lean_dec(x_21); +lean_dec(x_18); +lean_dec(x_8); lean_dec(x_7); -return x_13; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_97 = !lean_is_exclusive(x_24); +if (x_97 == 0) +{ +return x_24; } 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; uint8_t x_25; lean_object* x_26; uint8_t x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_14 = lean_ctor_get(x_7, 0); -x_15 = lean_ctor_get(x_7, 1); -x_16 = lean_ctor_get(x_7, 2); -x_17 = lean_ctor_get(x_7, 3); -x_18 = lean_ctor_get(x_7, 4); -x_19 = lean_ctor_get(x_7, 5); -x_20 = lean_ctor_get(x_7, 6); -x_21 = lean_ctor_get(x_7, 7); -x_22 = lean_ctor_get(x_7, 8); -x_23 = lean_ctor_get(x_7, 9); -x_24 = lean_ctor_get(x_7, 10); -x_25 = lean_ctor_get_uint8(x_7, sizeof(void*)*12); -x_26 = lean_ctor_get(x_7, 11); -x_27 = lean_ctor_get_uint8(x_7, sizeof(void*)*12 + 1); -lean_inc(x_26); -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_inc(x_15); -lean_inc(x_14); -lean_dec(x_7); -x_28 = l_Lean_replaceRef(x_1, x_19); -lean_dec(x_19); -x_29 = lean_alloc_ctor(0, 12, 2); -lean_ctor_set(x_29, 0, x_14); -lean_ctor_set(x_29, 1, x_15); -lean_ctor_set(x_29, 2, x_16); -lean_ctor_set(x_29, 3, x_17); -lean_ctor_set(x_29, 4, x_18); -lean_ctor_set(x_29, 5, x_28); -lean_ctor_set(x_29, 6, x_20); -lean_ctor_set(x_29, 7, x_21); -lean_ctor_set(x_29, 8, x_22); -lean_ctor_set(x_29, 9, x_23); -lean_ctor_set(x_29, 10, x_24); -lean_ctor_set(x_29, 11, x_26); -lean_ctor_set_uint8(x_29, sizeof(void*)*12, x_25); -lean_ctor_set_uint8(x_29, sizeof(void*)*12 + 1, x_27); -x_30 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__3(x_2, x_3, x_4, x_5, x_6, x_29, x_8, x_9); -lean_dec(x_29); -return x_30; +lean_object* x_98; lean_object* x_99; lean_object* x_100; +x_98 = lean_ctor_get(x_24, 0); +x_99 = lean_ctor_get(x_24, 1); +lean_inc(x_99); +lean_inc(x_98); +lean_dec(x_24); +x_100 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_100, 0, x_98); +lean_ctor_set(x_100, 1, x_99); +return x_100; } } } -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; -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_is_exclusive(x_12); -if (x_13 == 0) +} +else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; -x_14 = lean_ctor_get(x_12, 0); -x_15 = lean_ctor_get(x_12, 1); -x_16 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(x_14, x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_15); -lean_dec(x_2); -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_12, 1, x_18); -lean_ctor_set(x_12, 0, x_11); -lean_ctor_set_tag(x_16, 1); -lean_ctor_set(x_16, 0, x_12); -return x_16; -} -else +uint8_t x_108; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_108 = !lean_is_exclusive(x_10); +if (x_108 == 0) { -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_12, 1, x_19); -lean_ctor_set(x_12, 0, x_11); -x_21 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_21, 0, x_12); -lean_ctor_set(x_21, 1, x_20); -return x_21; -} +return x_10; } 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; -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 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(x_22, x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_23); -lean_dec(x_2); -x_25 = lean_ctor_get(x_24, 0); -lean_inc(x_25); -x_26 = lean_ctor_get(x_24, 1); -lean_inc(x_26); -if (lean_is_exclusive(x_24)) { - lean_ctor_release(x_24, 0); - lean_ctor_release(x_24, 1); - x_27 = x_24; -} else { - lean_dec_ref(x_24); - x_27 = lean_box(0); -} -x_28 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_28, 0, x_11); -lean_ctor_set(x_28, 1, x_25); -if (lean_is_scalar(x_27)) { - x_29 = lean_alloc_ctor(1, 2, 0); -} else { - x_29 = x_27; - lean_ctor_set_tag(x_29, 1); +lean_object* x_109; lean_object* x_110; lean_object* x_111; +x_109 = lean_ctor_get(x_10, 0); +x_110 = lean_ctor_get(x_10, 1); +lean_inc(x_110); +lean_inc(x_109); +lean_dec(x_10); +x_111 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_111, 0, x_109); +lean_ctor_set(x_111, 1, x_110); +return x_111; } -lean_ctor_set(x_29, 0, x_28); -lean_ctor_set(x_29, 1, x_26); -return x_29; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_structureSyntaxToView___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; -x_16 = lean_unsigned_to_nat(2u); -x_17 = l_Lean_Syntax_getArg(x_1, x_16); -x_18 = l_Lean_Syntax_getArgs(x_17); -lean_dec(x_17); -x_19 = lean_array_get_size(x_18); -x_20 = lean_unsigned_to_nat(0u); -x_21 = lean_nat_dec_lt(x_20, x_19); -if (x_21 == 0) -{ -lean_object* x_22; -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_9); +lean_object* x_10; +x_10 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_structureSyntaxToView___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_8); -lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_2); -lean_ctor_set(x_22, 1, x_15); -return x_22; +lean_dec(x_2); +return x_10; } -else -{ -uint8_t x_23; -x_23 = lean_nat_dec_le(x_19, x_19); -if (x_23 == 0) +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_structureSyntaxToView___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: { -lean_object* x_24; -lean_dec(x_19); -lean_dec(x_18); +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_foldlMUnsafe_fold___at_Lean_Elab_Command_structureSyntaxToView___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_11); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -x_24 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_24, 0, x_2); -lean_ctor_set(x_24, 1, x_15); -return x_24; -} -else -{ -size_t x_25; size_t x_26; lean_object* x_27; -x_25 = 0; -x_26 = lean_usize_of_nat(x_19); -lean_dec(x_19); -x_27 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1(x_3, x_4, x_5, x_6, x_7, x_8, x_18, x_25, x_26, x_2, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -lean_dec(x_18); -return x_27; -} -} -} -} -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("binderTactic", 12, 12); -return x_1; +lean_dec(x_2); +lean_dec(x_1); +return x_15; } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__2() { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_structureSyntaxToView___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]; _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__1; -x_2 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__2; -x_3 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__3; -x_4 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__1; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; +uint8_t x_19; lean_object* x_20; +x_19 = lean_unbox(x_5); +lean_dec(x_5); +x_20 = l_Lean_Elab_Command_structureSyntaxToView___lambda__1(x_1, x_2, x_3, x_4, x_19, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18); +return x_20; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6) { _start: { -lean_object* x_14; lean_object* x_15; uint8_t x_16; uint8_t x_17; -x_14 = lean_ctor_get(x_6, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_6, 1); -lean_inc(x_15); -lean_dec(x_6); -x_16 = 0; -x_17 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_404_(x_4, x_16); -if (x_17 == 0) +uint8_t x_7; +x_7 = lean_usize_dec_lt(x_5, x_4); +if (x_7 == 0) { -lean_object* x_18; lean_object* x_19; -x_18 = lean_box(0); -x_19 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__1(x_1, x_2, x_3, x_4, x_5, x_14, x_15, x_18, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -return x_19; +lean_inc(x_6); +return x_6; } else { -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; lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; -x_23 = lean_unsigned_to_nat(0u); -x_24 = l_Lean_Syntax_getArg(x_21, x_23); -lean_dec(x_21); -lean_inc(x_24); -x_25 = l_Lean_Syntax_getKind(x_24); -x_26 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__2; -x_27 = lean_name_eq(x_25, x_26); -lean_dec(x_25); -if (x_27 == 0) +lean_object* x_8; lean_object* x_9; uint8_t x_10; +x_8 = lean_array_uget(x_3, x_5); +x_9 = lean_ctor_get(x_8, 1); +lean_inc(x_9); +x_10 = lean_name_eq(x_9, x_1); +lean_dec(x_9); +if (x_10 == 0) { -lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_28 = lean_unsigned_to_nat(1u); -x_29 = l_Lean_Syntax_getArg(x_24, x_28); -lean_dec(x_24); -x_30 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_30, 0, x_29); -x_31 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__1(x_1, x_2, x_3, x_4, x_5, x_14, x_15, x_30, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -return x_31; -} -else +size_t x_11; size_t x_12; +lean_dec(x_8); +x_11 = 1; +x_12 = lean_usize_add(x_5, x_11); { -lean_object* x_32; lean_object* x_33; -lean_dec(x_24); -x_32 = lean_box(0); -x_33 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__1(x_1, x_2, x_3, x_4, x_5, x_14, x_15, x_32, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -return x_33; +size_t _tmp_4 = x_12; +lean_object* _tmp_5 = x_2; +x_5 = _tmp_4; +x_6 = _tmp_5; } +goto _start; } else { -lean_object* x_34; lean_object* x_35; -lean_dec(x_21); -x_34 = lean_box(0); -x_35 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__1(x_1, x_2, x_3, x_4, x_5, x_14, x_15, x_34, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -return x_35; +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_14 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_14, 0, x_8); +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_14); +x_16 = lean_box(0); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_15); +lean_ctor_set(x_17, 1, x_16); +return x_17; } } } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__1() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___lambda__1(lean_object* x_1) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("invalid field declaration, type must be provided when auto-param (tactic) is used", 81, 81); -return x_1; +lean_object* x_2; +x_2 = lean_box(0); +return x_2; } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__2() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___closed__1() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +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_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__3() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___closed__2() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("forall", 6, 6); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___lambda__1___boxed), 1, 0); return x_1; } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__4() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___closed__3() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__1; -x_2 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__2; -x_3 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__3; -x_4 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__3; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___closed__2; +x_2 = lean_box(0); +x_3 = lean_apply_1(x_1, x_2); +return x_3; } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__5() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("null", 4, 4); -return x_1; -} -} -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__5; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__7() { -_start: +size_t x_3; size_t x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_3 = lean_array_size(x_1); +x_4 = 0; +x_5 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___closed__1; +x_6 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___spec__1(x_2, x_5, x_1, x_3, x_4, x_5); +x_7 = lean_ctor_get(x_6, 0); +lean_inc(x_7); +lean_dec(x_6); +if (lean_obj_tag(x_7) == 0) { -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_8; +x_8 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___closed__3; +return x_8; } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__8() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("app", 3, 3); -return x_1; -} +lean_object* x_9; +x_9 = lean_ctor_get(x_7, 0); +lean_inc(x_9); +lean_dec(x_7); +return x_9; } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__9() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__1; -x_2 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__2; -x_3 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__3; -x_4 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__8; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__10() { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___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_1; -x_1 = lean_mk_string_unchecked("autoParam", 9, 9); -return x_1; +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___spec__1(x_1, x_2, x_3, x_7, x_8, x_6); +lean_dec(x_6); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_9; } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__11() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___lambda__1___boxed(lean_object* x_1) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__10; -x_2 = l_String_toSubstring_x27(x_1); +lean_object* x_2; +x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___lambda__1(x_1); +lean_dec(x_1); return x_2; } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__12() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___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(0); -x_2 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__10; -x_3 = l_Lean_Name_str___override(x_1, x_2); +lean_object* x_3; +x_3 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); return x_3; } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__13() { +LEAN_EXPORT uint8_t l___private_Lean_Elab_Structure_0__Lean_Elab_Command_containsFieldName(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(0); -x_2 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__12; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; -} +lean_object* x_3; +x_3 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f(x_1, x_2); +if (lean_obj_tag(x_3) == 0) +{ +uint8_t x_4; +x_4 = 0; +return x_4; } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__14() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__13; -x_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; +uint8_t x_5; +lean_dec(x_3); +x_5 = 1; +return x_5; +} } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__15() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_containsFieldName___boxed(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 = lean_box(2); -x_2 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__6; -x_3 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__7; -x_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); +uint8_t x_3; lean_object* x_4; +x_3 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_containsFieldName(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_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___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_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_replaceFieldInfo___spec__1(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { -uint8_t x_14; uint8_t x_15; -x_14 = 0; -x_15 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_404_(x_4, x_14); -if (x_15 == 0) +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_3, x_2); +if (x_5 == 0) { -lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; -x_16 = lean_unsigned_to_nat(3u); -x_17 = l_Lean_Syntax_getArg(x_1, x_16); -x_18 = l_Lean_Elab_expandDeclSig(x_17); -lean_dec(x_17); -x_19 = !lean_is_exclusive(x_18); -if (x_19 == 0) +lean_dec(x_1); +return x_4; +} +else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_18, 1); -x_21 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_21, 0, x_20); -lean_ctor_set(x_18, 1, x_21); -x_22 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2(x_1, x_2, x_3, x_4, x_5, x_18, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_12); -lean_dec(x_11); +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; size_t x_12; size_t x_13; +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_ctor_get(x_6, 1); +lean_inc(x_9); +x_10 = lean_ctor_get(x_1, 1); +lean_inc(x_10); +x_11 = lean_name_eq(x_9, x_10); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); -return x_22; +x_12 = 1; +x_13 = lean_usize_add(x_3, x_12); +if (x_11 == 0) +{ +lean_object* x_14; +x_14 = lean_array_uset(x_8, x_3, x_6); +x_3 = x_13; +x_4 = x_14; +goto _start; } 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_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, 1, 0); -lean_ctor_set(x_25, 0, x_24); -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_23); -lean_ctor_set(x_26, 1, x_25); -x_27 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2(x_1, x_2, x_3, x_4, x_5, x_26, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -return x_27; +lean_object* x_16; +lean_dec(x_6); +lean_inc(x_1); +x_16 = lean_array_uset(x_8, x_3, x_1); +x_3 = x_13; +x_4 = x_16; +goto _start; } } -else +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_replaceFieldInfo(lean_object* x_1, lean_object* x_2) { +_start: { -lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; -x_28 = lean_unsigned_to_nat(3u); -x_29 = l_Lean_Syntax_getArg(x_1, x_28); -x_30 = l_Lean_Elab_expandOptDeclSig(x_29); -lean_dec(x_29); -x_31 = !lean_is_exclusive(x_30); -if (x_31 == 0) +size_t x_3; size_t x_4; lean_object* x_5; +x_3 = lean_array_size(x_1); +x_4 = 0; +x_5 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_replaceFieldInfo___spec__1(x_2, x_3, x_4, x_1); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_replaceFieldInfo___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: { -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; -x_32 = lean_ctor_get(x_30, 0); -x_33 = lean_ctor_get(x_30, 1); -x_34 = lean_unsigned_to_nat(4u); -x_35 = l_Lean_Syntax_getArg(x_1, x_34); -x_36 = l_Lean_Syntax_isNone(x_35); -if (x_36 == 0) +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_Elab_Structure_0__Lean_Elab_Command_replaceFieldInfo___spec__1(x_1, x_5, x_6, x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: { -lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; -x_37 = lean_unsigned_to_nat(0u); -x_38 = l_Lean_Syntax_getArg(x_35, x_37); -lean_dec(x_35); -lean_inc(x_38); -x_39 = l_Lean_Syntax_getKind(x_38); -x_40 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__2; -x_41 = lean_name_eq(x_39, x_40); -lean_dec(x_39); -if (x_41 == 0) +uint8_t x_10; +x_10 = lean_usize_dec_lt(x_5, x_4); +if (x_10 == 0) { -lean_object* x_42; -lean_dec(x_38); -x_42 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2(x_1, x_2, x_3, x_4, x_5, x_30, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -return x_42; +lean_object* x_11; +lean_dec(x_2); +x_11 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_11, 0, x_6); +lean_ctor_set(x_11, 1, x_9); +return x_11; } else { -if (lean_obj_tag(x_33) == 0) +lean_object* x_12; uint8_t x_13; +lean_dec(x_6); +x_12 = lean_array_uget(x_3, x_5); +x_13 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_containsFieldName(x_1, x_12); +if (x_13 == 0) { -lean_object* x_43; lean_object* x_44; uint8_t x_45; -lean_free_object(x_30); -lean_dec(x_32); -lean_dec(x_5); -lean_dec(x_3); -lean_dec(x_2); -x_43 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__2; -x_44 = l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__2(x_38, x_43, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +size_t x_14; size_t x_15; lean_dec(x_12); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_38); -x_45 = !lean_is_exclusive(x_44); -if (x_45 == 0) -{ -return x_44; -} -else +x_14 = 1; +x_15 = lean_usize_add(x_5, x_14); +lean_inc(x_2); { -lean_object* x_46; lean_object* x_47; lean_object* x_48; -x_46 = lean_ctor_get(x_44, 0); -x_47 = lean_ctor_get(x_44, 1); -lean_inc(x_47); -lean_inc(x_46); -lean_dec(x_44); -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; +size_t _tmp_4 = x_15; +lean_object* _tmp_5 = x_2; +x_5 = _tmp_4; +x_6 = _tmp_5; } +goto _start; } else { -uint8_t x_49; -x_49 = !lean_is_exclusive(x_33); -if (x_49 == 0) -{ -lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; -x_50 = lean_ctor_get(x_33, 0); -x_51 = lean_unsigned_to_nat(2u); -x_52 = l_Lean_Syntax_getArg(x_38, x_51); -lean_dec(x_38); -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_52); -x_53 = l_Lean_Elab_Term_declareTacticSyntax(x_52, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_53) == 0) -{ -lean_object* x_54; lean_object* x_55; lean_object* x_56; uint8_t x_57; lean_object* x_58; lean_object* x_59; uint8_t x_60; -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_ctor_get(x_11, 5); -lean_inc(x_56); -x_57 = 0; -x_58 = l_Lean_SourceInfo_fromRef(x_56, x_57); -lean_dec(x_56); -x_59 = lean_st_ref_get(x_12, x_55); -x_60 = !lean_is_exclusive(x_59); -if (x_60 == 0) -{ -lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; 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; -x_61 = lean_ctor_get(x_59, 1); -x_62 = lean_ctor_get(x_59, 0); -lean_dec(x_62); -x_63 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__3; -lean_inc(x_58); -lean_ctor_set_tag(x_59, 2); -lean_ctor_set(x_59, 1, x_63); -lean_ctor_set(x_59, 0, x_58); -x_64 = l_Lean_Syntax_getArgs(x_32); -lean_dec(x_32); -x_65 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__7; -x_66 = l_Array_append___rarg(x_65, x_64); -lean_dec(x_64); -x_67 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__6; -lean_inc(x_58); -x_68 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_68, 0, x_58); -lean_ctor_set(x_68, 1, x_67); -lean_ctor_set(x_68, 2, x_66); -lean_inc(x_58); -x_69 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_69, 0, x_58); -lean_ctor_set(x_69, 1, x_67); -lean_ctor_set(x_69, 2, x_65); -x_70 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__8; -lean_inc(x_58); -x_71 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_71, 0, x_58); -lean_ctor_set(x_71, 1, x_70); -x_72 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__4; -lean_inc(x_58); -x_73 = l_Lean_Syntax_node5(x_58, x_72, x_59, x_68, x_69, x_71, x_50); -x_74 = lean_ctor_get(x_11, 10); -lean_inc(x_74); -x_75 = lean_st_ref_get(x_12, x_61); -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_ctor_get(x_76, 0); -lean_inc(x_78); -lean_dec(x_76); -x_79 = lean_environment_main_module(x_78); -x_80 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__12; -x_81 = l_Lean_addMacroScope(x_79, x_80, x_74); -x_82 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__11; -x_83 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__14; -lean_inc(x_58); -x_84 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_84, 0, x_58); -lean_ctor_set(x_84, 1, x_82); -lean_ctor_set(x_84, 2, x_81); -lean_ctor_set(x_84, 3, x_83); -x_85 = l_Lean_mkIdentFrom(x_52, x_54, x_57); -lean_dec(x_52); -lean_inc(x_58); -x_86 = l_Lean_Syntax_node2(x_58, x_67, x_73, x_85); -x_87 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__9; -x_88 = l_Lean_Syntax_node2(x_58, x_87, x_84, x_86); -lean_ctor_set(x_33, 0, x_88); -x_89 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__15; -lean_ctor_set(x_30, 0, x_89); -x_90 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2(x_1, x_2, x_3, x_4, x_5, x_30, x_7, x_8, x_9, x_10, x_11, x_12, x_77); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -return x_90; +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +lean_dec(x_2); +x_17 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_17, 0, x_12); +x_18 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_18, 0, x_17); +x_19 = lean_box(0); +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_18); +lean_ctor_set(x_20, 1, x_19); +x_21 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_21, 0, x_20); +lean_ctor_set(x_21, 1, x_9); +return x_21; } -else +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f___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_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; -x_91 = lean_ctor_get(x_59, 1); -lean_inc(x_91); -lean_dec(x_59); -x_92 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__3; -lean_inc(x_58); -x_93 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_93, 0, x_58); -lean_ctor_set(x_93, 1, x_92); -x_94 = l_Lean_Syntax_getArgs(x_32); -lean_dec(x_32); -x_95 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__7; -x_96 = l_Array_append___rarg(x_95, x_94); -lean_dec(x_94); -x_97 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__6; -lean_inc(x_58); -x_98 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_98, 0, x_58); -lean_ctor_set(x_98, 1, x_97); -lean_ctor_set(x_98, 2, x_96); -lean_inc(x_58); -x_99 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_99, 0, x_58); -lean_ctor_set(x_99, 1, x_97); -lean_ctor_set(x_99, 2, x_95); -x_100 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__8; -lean_inc(x_58); -x_101 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_101, 0, x_58); -lean_ctor_set(x_101, 1, x_100); -x_102 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__4; -lean_inc(x_58); -x_103 = l_Lean_Syntax_node5(x_58, x_102, x_93, x_98, x_99, x_101, x_50); -x_104 = lean_ctor_get(x_11, 10); -lean_inc(x_104); -x_105 = lean_st_ref_get(x_12, x_91); -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_environment_main_module(x_108); -x_110 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__12; -x_111 = l_Lean_addMacroScope(x_109, x_110, x_104); -x_112 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__11; -x_113 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__14; -lean_inc(x_58); -x_114 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_114, 0, x_58); -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 = l_Lean_mkIdentFrom(x_52, x_54, x_57); -lean_dec(x_52); -lean_inc(x_58); -x_116 = l_Lean_Syntax_node2(x_58, x_97, x_103, x_115); -x_117 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__9; -x_118 = l_Lean_Syntax_node2(x_58, x_117, x_114, x_116); -lean_ctor_set(x_33, 0, x_118); -x_119 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__15; -lean_ctor_set(x_30, 0, x_119); -x_120 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2(x_1, x_2, x_3, x_4, x_5, x_30, x_7, x_8, x_9, x_10, x_11, x_12, x_107); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -return x_120; +lean_object* x_6; +x_6 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_6, 0, x_1); +lean_ctor_set(x_6, 1, x_5); +return x_6; } } -else +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: { -uint8_t x_121; -lean_dec(x_52); -lean_free_object(x_33); -lean_dec(x_50); -lean_free_object(x_30); -lean_dec(x_32); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; lean_object* x_11; lean_object* x_12; 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_6 = lean_st_ref_get(x_4, x_5); +x_7 = lean_ctor_get(x_6, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_6, 1); +lean_inc(x_8); +lean_dec(x_6); +x_9 = lean_ctor_get(x_7, 0); +lean_inc(x_9); lean_dec(x_7); -lean_dec(x_5); -lean_dec(x_3); -lean_dec(x_2); -x_121 = !lean_is_exclusive(x_53); -if (x_121 == 0) +x_10 = 1; +x_11 = l_Lean_getStructureFieldsFlattened(x_9, x_2, x_10); +lean_dec(x_9); +x_12 = lean_box(0); +x_13 = lean_array_size(x_11); +x_14 = 0; +x_15 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___closed__1; +x_16 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f___spec__1(x_1, x_15, x_11, x_13, x_14, x_15, x_3, x_4, x_8); +lean_dec(x_11); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +lean_dec(x_17); +if (lean_obj_tag(x_18) == 0) { -return x_53; +uint8_t x_19; +x_19 = !lean_is_exclusive(x_16); +if (x_19 == 0) +{ +lean_object* x_20; +x_20 = lean_ctor_get(x_16, 0); +lean_dec(x_20); +lean_ctor_set(x_16, 0, x_12); +return x_16; } else { -lean_object* x_122; lean_object* x_123; lean_object* x_124; -x_122 = lean_ctor_get(x_53, 0); -x_123 = lean_ctor_get(x_53, 1); -lean_inc(x_123); -lean_inc(x_122); -lean_dec(x_53); -x_124 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_124, 0, x_122); -lean_ctor_set(x_124, 1, x_123); -return x_124; -} +lean_object* x_21; lean_object* x_22; +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_12); +lean_ctor_set(x_22, 1, x_21); +return x_22; } } else { -lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; -x_125 = lean_ctor_get(x_33, 0); -lean_inc(x_125); -lean_dec(x_33); -x_126 = lean_unsigned_to_nat(2u); -x_127 = l_Lean_Syntax_getArg(x_38, x_126); -lean_dec(x_38); -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_127); -x_128 = l_Lean_Elab_Term_declareTacticSyntax(x_127, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_128) == 0) +uint8_t x_23; +x_23 = !lean_is_exclusive(x_16); +if (x_23 == 0) { -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; 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_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_11, 5); -lean_inc(x_131); -x_132 = 0; -x_133 = l_Lean_SourceInfo_fromRef(x_131, x_132); -lean_dec(x_131); -x_134 = lean_st_ref_get(x_12, x_130); -x_135 = lean_ctor_get(x_134, 1); -lean_inc(x_135); -if (lean_is_exclusive(x_134)) { - lean_ctor_release(x_134, 0); - lean_ctor_release(x_134, 1); - x_136 = x_134; -} else { - lean_dec_ref(x_134); - x_136 = lean_box(0); -} -x_137 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__3; -lean_inc(x_133); -if (lean_is_scalar(x_136)) { - x_138 = lean_alloc_ctor(2, 2, 0); -} else { - x_138 = x_136; - lean_ctor_set_tag(x_138, 2); -} -lean_ctor_set(x_138, 0, x_133); -lean_ctor_set(x_138, 1, x_137); -x_139 = l_Lean_Syntax_getArgs(x_32); -lean_dec(x_32); -x_140 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__7; -x_141 = l_Array_append___rarg(x_140, x_139); -lean_dec(x_139); -x_142 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__6; -lean_inc(x_133); -x_143 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_143, 0, x_133); -lean_ctor_set(x_143, 1, x_142); -lean_ctor_set(x_143, 2, x_141); -lean_inc(x_133); -x_144 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_144, 0, x_133); -lean_ctor_set(x_144, 1, x_142); -lean_ctor_set(x_144, 2, x_140); -x_145 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__8; -lean_inc(x_133); -x_146 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_146, 0, x_133); -lean_ctor_set(x_146, 1, x_145); -x_147 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__4; -lean_inc(x_133); -x_148 = l_Lean_Syntax_node5(x_133, x_147, x_138, x_143, x_144, x_146, x_125); -x_149 = lean_ctor_get(x_11, 10); -lean_inc(x_149); -x_150 = lean_st_ref_get(x_12, x_135); -x_151 = lean_ctor_get(x_150, 0); -lean_inc(x_151); -x_152 = lean_ctor_get(x_150, 1); -lean_inc(x_152); -lean_dec(x_150); -x_153 = lean_ctor_get(x_151, 0); -lean_inc(x_153); -lean_dec(x_151); -x_154 = lean_environment_main_module(x_153); -x_155 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__12; -x_156 = l_Lean_addMacroScope(x_154, x_155, x_149); -x_157 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__11; -x_158 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__14; -lean_inc(x_133); -x_159 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_159, 0, x_133); -lean_ctor_set(x_159, 1, x_157); -lean_ctor_set(x_159, 2, x_156); -lean_ctor_set(x_159, 3, x_158); -x_160 = l_Lean_mkIdentFrom(x_127, x_129, x_132); -lean_dec(x_127); -lean_inc(x_133); -x_161 = l_Lean_Syntax_node2(x_133, x_142, x_148, x_160); -x_162 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__9; -x_163 = l_Lean_Syntax_node2(x_133, x_162, x_159, x_161); -x_164 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_164, 0, x_163); -x_165 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__15; -lean_ctor_set(x_30, 1, x_164); -lean_ctor_set(x_30, 0, x_165); -x_166 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2(x_1, x_2, x_3, x_4, x_5, x_30, x_7, x_8, x_9, x_10, x_11, x_12, x_152); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -return x_166; +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_16, 0); +lean_dec(x_24); +x_25 = lean_ctor_get(x_18, 0); +lean_inc(x_25); +lean_dec(x_18); +lean_ctor_set(x_16, 0, x_25); +return x_16; } else { -lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; -lean_dec(x_127); -lean_dec(x_125); -lean_free_object(x_30); -lean_dec(x_32); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_5); -lean_dec(x_3); -lean_dec(x_2); -x_167 = lean_ctor_get(x_128, 0); -lean_inc(x_167); -x_168 = lean_ctor_get(x_128, 1); -lean_inc(x_168); -if (lean_is_exclusive(x_128)) { - lean_ctor_release(x_128, 0); - lean_ctor_release(x_128, 1); - x_169 = x_128; -} else { - lean_dec_ref(x_128); - x_169 = lean_box(0); -} -if (lean_is_scalar(x_169)) { - x_170 = lean_alloc_ctor(1, 2, 0); -} else { - x_170 = x_169; -} -lean_ctor_set(x_170, 0, x_167); -lean_ctor_set(x_170, 1, x_168); -return x_170; -} +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_16, 1); +lean_inc(x_26); +lean_dec(x_16); +x_27 = lean_ctor_get(x_18, 0); +lean_inc(x_27); +lean_dec(x_18); +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_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: { -lean_object* x_171; -lean_dec(x_35); -x_171 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2(x_1, x_2, x_3, x_4, x_5, x_30, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); +size_t x_10; size_t x_11; lean_object* x_12; +x_10 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_11 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_12 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f___spec__1(x_1, x_2, x_3, x_10, x_11, x_6, x_7, x_8, x_9); lean_dec(x_8); -return x_171; -} +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_1); +return x_12; } -else -{ -lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; uint8_t x_176; -x_172 = lean_ctor_get(x_30, 0); -x_173 = lean_ctor_get(x_30, 1); -lean_inc(x_173); -lean_inc(x_172); -lean_dec(x_30); -x_174 = lean_unsigned_to_nat(4u); -x_175 = l_Lean_Syntax_getArg(x_1, x_174); -x_176 = l_Lean_Syntax_isNone(x_175); -if (x_176 == 0) -{ -lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; uint8_t x_181; -x_177 = lean_unsigned_to_nat(0u); -x_178 = l_Lean_Syntax_getArg(x_175, x_177); -lean_dec(x_175); -lean_inc(x_178); -x_179 = l_Lean_Syntax_getKind(x_178); -x_180 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__2; -x_181 = lean_name_eq(x_179, x_180); -lean_dec(x_179); -if (x_181 == 0) -{ -lean_object* x_182; lean_object* x_183; -lean_dec(x_178); -x_182 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_182, 0, x_172); -lean_ctor_set(x_182, 1, x_173); -x_183 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2(x_1, x_2, x_3, x_4, x_5, x_182, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -return x_183; } -else -{ -if (lean_obj_tag(x_173) == 0) +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f___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_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; -lean_dec(x_172); -lean_dec(x_5); +lean_object* x_6; +x_6 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f___lambda__1(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_184 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__2; -x_185 = l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__2(x_178, x_184, 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_178); -x_186 = lean_ctor_get(x_185, 0); -lean_inc(x_186); -x_187 = lean_ctor_get(x_185, 1); -lean_inc(x_187); -if (lean_is_exclusive(x_185)) { - lean_ctor_release(x_185, 0); - lean_ctor_release(x_185, 1); - x_188 = x_185; -} else { - lean_dec_ref(x_185); - x_188 = lean_box(0); +return x_6; } -if (lean_is_scalar(x_188)) { - x_189 = lean_alloc_ctor(1, 2, 0); -} else { - x_189 = x_188; } -lean_ctor_set(x_189, 0, x_186); -lean_ctor_set(x_189, 1, x_187); -return x_189; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; +x_6 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +return x_6; } -else +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +_start: { -lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; -x_190 = lean_ctor_get(x_173, 0); -lean_inc(x_190); -if (lean_is_exclusive(x_173)) { - lean_ctor_release(x_173, 0); - x_191 = x_173; -} else { - lean_dec_ref(x_173); - x_191 = lean_box(0); +lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; +lean_inc(x_2); +lean_inc(x_1); +x_17 = l_Lean_Name_append(x_1, x_2); +x_18 = lean_ctor_get(x_14, 5); +lean_inc(x_18); +x_19 = lean_box(0); +x_20 = 2; +x_21 = lean_alloc_ctor(0, 5, 1); +lean_ctor_set(x_21, 0, x_18); +lean_ctor_set(x_21, 1, x_2); +lean_ctor_set(x_21, 2, x_17); +lean_ctor_set(x_21, 3, x_9); +lean_ctor_set(x_21, 4, x_19); +lean_ctor_set_uint8(x_21, sizeof(void*)*5, x_20); +x_22 = lean_array_push(x_3, x_21); +x_23 = lean_unsigned_to_nat(1u); +x_24 = lean_nat_add(x_4, x_23); +x_25 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg(x_1, x_5, x_6, x_7, x_8, x_24, x_22, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +return x_25; } -x_192 = lean_unsigned_to_nat(2u); -x_193 = l_Lean_Syntax_getArg(x_178, x_192); -lean_dec(x_178); +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_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, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +_start: +{ +lean_object* x_17; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_193); -x_194 = l_Lean_Elab_Term_declareTacticSyntax(x_193, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_194) == 0) +lean_inc(x_2); +lean_inc(x_1); +x_17 = l_Lean_Meta_mkProjection(x_1, x_2, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_17) == 0) { -lean_object* x_195; lean_object* x_196; lean_object* x_197; uint8_t x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_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; -x_195 = lean_ctor_get(x_194, 0); -lean_inc(x_195); -x_196 = lean_ctor_get(x_194, 1); -lean_inc(x_196); -lean_dec(x_194); -x_197 = lean_ctor_get(x_11, 5); -lean_inc(x_197); -x_198 = 0; -x_199 = l_Lean_SourceInfo_fromRef(x_197, x_198); -lean_dec(x_197); -x_200 = lean_st_ref_get(x_12, x_196); -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_200); - x_202 = lean_box(0); -} -x_203 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__3; -lean_inc(x_199); -if (lean_is_scalar(x_202)) { - x_204 = lean_alloc_ctor(2, 2, 0); -} else { - x_204 = x_202; - lean_ctor_set_tag(x_204, 2); -} -lean_ctor_set(x_204, 0, x_199); -lean_ctor_set(x_204, 1, x_203); -x_205 = l_Lean_Syntax_getArgs(x_172); -lean_dec(x_172); -x_206 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__7; -x_207 = l_Array_append___rarg(x_206, x_205); -lean_dec(x_205); -x_208 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__6; -lean_inc(x_199); -x_209 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_209, 0, x_199); -lean_ctor_set(x_209, 1, x_208); -lean_ctor_set(x_209, 2, x_207); -lean_inc(x_199); -x_210 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_210, 0, x_199); -lean_ctor_set(x_210, 1, x_208); -lean_ctor_set(x_210, 2, x_206); -x_211 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__8; -lean_inc(x_199); -x_212 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_212, 0, x_199); -lean_ctor_set(x_212, 1, x_211); -x_213 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__4; -lean_inc(x_199); -x_214 = l_Lean_Syntax_node5(x_199, x_213, x_204, x_209, x_210, x_212, x_190); -x_215 = lean_ctor_get(x_11, 10); -lean_inc(x_215); -x_216 = lean_st_ref_get(x_12, x_201); -x_217 = lean_ctor_get(x_216, 0); -lean_inc(x_217); -x_218 = lean_ctor_get(x_216, 1); -lean_inc(x_218); -lean_dec(x_216); -x_219 = lean_ctor_get(x_217, 0); -lean_inc(x_219); -lean_dec(x_217); -x_220 = lean_environment_main_module(x_219); -x_221 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__12; -x_222 = l_Lean_addMacroScope(x_220, x_221, x_215); -x_223 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__11; -x_224 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__14; -lean_inc(x_199); -x_225 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_225, 0, x_199); -lean_ctor_set(x_225, 1, x_223); -lean_ctor_set(x_225, 2, x_222); -lean_ctor_set(x_225, 3, x_224); -x_226 = l_Lean_mkIdentFrom(x_193, x_195, x_198); -lean_dec(x_193); -lean_inc(x_199); -x_227 = l_Lean_Syntax_node2(x_199, x_208, x_214, x_226); -x_228 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__9; -x_229 = l_Lean_Syntax_node2(x_199, x_228, x_225, x_227); -if (lean_is_scalar(x_191)) { - x_230 = lean_alloc_ctor(1, 1, 0); -} else { - x_230 = x_191; -} -lean_ctor_set(x_230, 0, x_229); -x_231 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__15; -x_232 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_232, 0, x_231); -lean_ctor_set(x_232, 1, x_230); -x_233 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2(x_1, x_2, x_3, x_4, x_5, x_232, x_7, x_8, x_9, x_10, x_11, x_12, x_218); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -return x_233; +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); +lean_dec(x_17); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_18); +x_20 = lean_infer_type(x_18, x_12, x_13, x_14, x_15, x_19); +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; +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +lean_inc(x_2); +x_23 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___lambda__1___boxed), 16, 8); +lean_closure_set(x_23, 0, x_3); +lean_closure_set(x_23, 1, x_2); +lean_closure_set(x_23, 2, x_4); +lean_closure_set(x_23, 3, x_5); +lean_closure_set(x_23, 4, x_1); +lean_closure_set(x_23, 5, x_6); +lean_closure_set(x_23, 6, x_7); +lean_closure_set(x_23, 7, x_8); +x_24 = 0; +x_25 = l_Lean_Meta_withLetDecl___at_Lean_Elab_Term_elabLetDeclAux___spec__2___rarg(x_2, x_21, x_18, x_23, x_24, x_10, x_11, x_12, x_13, x_14, x_15, x_22); +return x_25; } else { -lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; -lean_dec(x_193); -lean_dec(x_191); -lean_dec(x_190); -lean_dec(x_172); +uint8_t x_26; +lean_dec(x_18); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); -lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); +lean_dec(x_6); lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_234 = lean_ctor_get(x_194, 0); -lean_inc(x_234); -x_235 = lean_ctor_get(x_194, 1); -lean_inc(x_235); -if (lean_is_exclusive(x_194)) { - lean_ctor_release(x_194, 0); - lean_ctor_release(x_194, 1); - x_236 = x_194; -} else { - lean_dec_ref(x_194); - x_236 = lean_box(0); -} -if (lean_is_scalar(x_236)) { - x_237 = lean_alloc_ctor(1, 2, 0); -} else { - x_237 = x_236; -} -lean_ctor_set(x_237, 0, x_234); -lean_ctor_set(x_237, 1, x_235); -return x_237; +lean_dec(x_1); +x_26 = !lean_is_exclusive(x_20); +if (x_26 == 0) +{ +return x_20; } +else +{ +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_dec(x_20); +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_27); +lean_ctor_set(x_29, 1, x_28); +return x_29; } } } else { -lean_object* x_238; lean_object* x_239; -lean_dec(x_175); -x_238 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_238, 0, x_172); -lean_ctor_set(x_238, 1, x_173); -x_239 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2(x_1, x_2, x_3, x_4, x_5, x_238, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +uint8_t x_30; +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); -return x_239; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_30 = !lean_is_exclusive(x_17); +if (x_30 == 0) +{ +return x_17; } +else +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_31 = lean_ctor_get(x_17, 0); +x_32 = lean_ctor_get(x_17, 1); +lean_inc(x_32); +lean_inc(x_31); +lean_dec(x_17); +x_33 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_33, 0, x_31); +lean_ctor_set(x_33, 1, x_32); +return x_33; } } } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4___closed__1() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("invalid 'protected' field in a 'private' structure", 50, 50); +x_1 = lean_mk_string_unchecked("field '", 7, 7); return x_1; } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4___closed__2() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4___closed__1; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4(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) { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__3() { _start: { -uint8_t x_15; -x_15 = l_Lean_Elab_Modifiers_isProtected(x_5); -if (x_15 == 0) -{ -lean_object* x_16; lean_object* x_17; -x_16 = lean_box(0); -x_17 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3(x_1, x_2, x_3, x_4, x_5, x_16, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -return x_17; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("' from '", 8, 8); +return x_1; } -else -{ -uint8_t x_18; -x_18 = l_Lean_Elab_Modifiers_isPrivate(x_6); -if (x_18 == 0) -{ -lean_object* x_19; lean_object* x_20; -x_19 = lean_box(0); -x_20 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3(x_1, x_2, x_3, x_4, x_5, x_19, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -return x_20; } -else +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__4() { +_start: { -lean_object* x_21; lean_object* x_22; uint8_t x_23; -lean_dec(x_5); -lean_dec(x_3); -lean_dec(x_2); -x_21 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4___closed__2; -x_22 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_21, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -x_23 = !lean_is_exclusive(x_22); -if (x_23 == 0) -{ -return x_22; -} -else -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_22, 0); -x_25 = lean_ctor_get(x_22, 1); -lean_inc(x_25); -lean_inc(x_24); -lean_dec(x_22); -x_26 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_26, 0, x_24); -lean_ctor_set(x_26, 1, x_25); -return x_26; -} -} -} +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__1() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__5() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("invalid 'private' field in a 'private' structure", 48, 48); +x_1 = lean_mk_string_unchecked("' has already been declared", 27, 27); return x_1; } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__2() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__6() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__1; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__5; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5(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_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Syntax_getArg(x_1, x_13); -lean_inc(x_10); -lean_inc(x_6); -x_15 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1(x_14, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_14); -if (lean_obj_tag(x_15) == 0) -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; -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_object* x_15; uint8_t x_16; +x_15 = lean_array_get_size(x_4); +x_16 = lean_nat_dec_lt(x_6, x_15); lean_dec(x_15); -lean_inc(x_6); -x_18 = l_Lean_Elab_Command_checkValidFieldModifier(x_16, x_6, x_7, x_8, x_9, x_10, x_11, x_17); -if (lean_obj_tag(x_18) == 0) -{ -lean_object* x_19; uint8_t x_20; -x_19 = lean_ctor_get(x_18, 1); -lean_inc(x_19); -lean_dec(x_18); -x_20 = l_Lean_Elab_Modifiers_isPrivate(x_16); -if (x_20 == 0) -{ -lean_object* x_21; lean_object* x_22; -x_21 = lean_box(0); -x_22 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4(x_1, x_2, x_3, x_5, x_16, x_4, x_21, x_6, x_7, x_8, x_9, x_10, x_11, x_19); -return x_22; -} -else -{ -uint8_t x_23; -x_23 = l_Lean_Elab_Modifiers_isPrivate(x_4); -if (x_23 == 0) -{ -lean_object* x_24; lean_object* x_25; -x_24 = lean_box(0); -x_25 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4(x_1, x_2, x_3, x_5, x_16, x_4, x_24, x_6, x_7, x_8, x_9, x_10, x_11, x_19); -return x_25; -} -else +if (x_16 == 0) { -lean_object* x_26; lean_object* x_27; uint8_t x_28; -lean_dec(x_16); +lean_object* x_17; +lean_dec(x_6); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_26 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__2; -x_27 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_26, x_6, x_7, x_8, x_9, x_10, x_11, x_19); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -x_28 = !lean_is_exclusive(x_27); -if (x_28 == 0) -{ -return x_27; +lean_dec(x_1); +x_17 = lean_apply_8(x_5, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +return x_17; } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_27, 0); -x_30 = lean_ctor_get(x_27, 1); -lean_inc(x_30); -lean_inc(x_29); -lean_dec(x_27); -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_18; uint8_t x_19; +x_18 = lean_array_fget(x_4, x_6); +x_19 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_containsFieldName(x_7, x_18); +if (x_19 == 0) +{ +lean_object* x_20; lean_object* x_21; +x_20 = lean_box(0); +x_21 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___lambda__2(x_2, x_18, x_1, x_7, x_6, x_3, x_4, x_5, x_20, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +return x_21; } else { -uint8_t x_32; -lean_dec(x_16); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); +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_dec(x_7); lean_dec(x_6); -lean_dec(x_3); +lean_dec(x_5); +lean_dec(x_4); lean_dec(x_2); -x_32 = !lean_is_exclusive(x_18); +lean_dec(x_1); +x_22 = l_Lean_MessageData_ofName(x_18); +x_23 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__2; +x_24 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_24, 0, x_23); +lean_ctor_set(x_24, 1, x_22); +x_25 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__4; +x_26 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_26, 0, x_24); +lean_ctor_set(x_26, 1, x_25); +x_27 = l_Lean_MessageData_ofName(x_3); +x_28 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +x_29 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__6; +x_30 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +x_31 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_30, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +x_32 = !lean_is_exclusive(x_31); if (x_32 == 0) { -return x_18; +return x_31; } else { lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_33 = lean_ctor_get(x_18, 0); -x_34 = lean_ctor_get(x_18, 1); +x_33 = lean_ctor_get(x_31, 0); +x_34 = lean_ctor_get(x_31, 1); lean_inc(x_34); lean_inc(x_33); -lean_dec(x_18); +lean_dec(x_31); x_35 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_35, 0, x_33); lean_ctor_set(x_35, 1, x_34); @@ -8901,2302 +8594,2205 @@ return x_35; } } } -else -{ -uint8_t x_36; -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_3); -lean_dec(x_2); -x_36 = !lean_is_exclusive(x_15); -if (x_36 == 0) -{ -return x_15; -} -else -{ -lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_37 = lean_ctor_get(x_15, 0); -x_38 = lean_ctor_get(x_15, 1); -lean_inc(x_38); -lean_inc(x_37); -lean_dec(x_15); -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; -} -} } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__1() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go(lean_object* x_1) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("structExplicitBinder", 20, 20); -return x_1; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg), 14, 0); +return x_2; } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__2() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__1; -x_2 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__2; -x_3 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__1; -x_4 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__1; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; +lean_object* x_17; +x_17 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +lean_dec(x_4); +return x_17; } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__3() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___lambda__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_1; -x_1 = lean_mk_string_unchecked("structImplicitBinder", 20, 20); -return x_1; +lean_object* x_17; +x_17 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +lean_dec(x_9); +return x_17; } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__4() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields___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) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__1; -x_2 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__2; -x_3 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__1; -x_4 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__3; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; +lean_object* x_14; lean_object* x_15; +x_14 = lean_unsigned_to_nat(0u); +x_15 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg(x_1, x_2, x_3, x_4, x_6, x_14, x_5, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +return x_15; } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__5() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields(lean_object* x_1) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("structInstBinder", 16, 16); -return x_1; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields___rarg), 13, 0); +return x_2; } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__6() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getNestedProjectionArg___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_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__1; -x_2 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__2; -x_3 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__1; -x_4 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__5; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; +lean_object* x_8; +x_8 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_8, 0, x_1); +lean_ctor_set(x_8, 1, x_7); +return x_8; } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__7() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getNestedProjectionArg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("unexpected kind of structure field", 34, 34); -return x_1; -} -} -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__8() { -_start: +lean_object* x_7; +x_7 = l_Lean_Expr_getAppFn(x_1); +if (lean_obj_tag(x_7) == 4) { -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__7; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} +lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_8 = lean_ctor_get(x_7, 0); +lean_inc(x_8); +lean_dec(x_7); +x_9 = l_Lean_getProjectionFnInfo_x3f___at_Lean_Meta_getStuckMVar_x3f___spec__1(x_8, x_2, x_3, x_4, x_5, x_6); +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; +x_12 = lean_ctor_get(x_9, 0); +lean_dec(x_12); +lean_ctor_set(x_9, 0, x_1); +return x_9; } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___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: +else { -lean_object* x_13; lean_object* x_14; uint8_t x_15; -lean_inc(x_4); -x_13 = l_Lean_Syntax_getKind(x_4); -x_14 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__2; -x_15 = lean_name_eq(x_13, x_14); -if (x_15 == 0) +lean_object* x_13; lean_object* x_14; +x_13 = lean_ctor_get(x_9, 1); +lean_inc(x_13); +lean_dec(x_9); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_1); +lean_ctor_set(x_14, 1, x_13); +return x_14; +} +} +else { -lean_object* x_16; uint8_t x_17; -x_16 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__4; -x_17 = lean_name_eq(x_13, x_16); -if (x_17 == 0) +lean_object* x_15; uint8_t x_16; +x_15 = lean_ctor_get(x_10, 0); +lean_inc(x_15); +lean_dec(x_10); +x_16 = !lean_is_exclusive(x_9); +if (x_16 == 0) { -lean_object* x_18; uint8_t x_19; -x_18 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__6; -x_19 = lean_name_eq(x_13, x_18); -lean_dec(x_13); -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; lean_object* x_23; uint8_t x_24; +x_17 = lean_ctor_get(x_9, 1); +x_18 = lean_ctor_get(x_9, 0); +lean_dec(x_18); +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___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); +x_24 = lean_nat_dec_eq(x_21, x_23); +lean_dec(x_23); +lean_dec(x_21); +if (x_24 == 0) { -lean_object* x_20; lean_object* x_21; uint8_t x_22; -lean_dec(x_4); -lean_dec(x_2); +lean_ctor_set(x_9, 0, x_1); +return x_9; +} +else +{ +lean_object* x_25; lean_object* x_26; uint8_t x_27; +lean_free_object(x_9); +x_25 = l_Lean_Expr_appArg_x21(x_1); lean_dec(x_1); -x_20 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__8; -x_21 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__4(x_20, 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); -x_22 = !lean_is_exclusive(x_21); -if (x_22 == 0) +x_26 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getNestedProjectionArg(x_25, x_2, x_3, x_4, x_5, x_17); +x_27 = !lean_is_exclusive(x_26); +if (x_27 == 0) { -return x_21; +return x_26; } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_21, 0); -x_24 = lean_ctor_get(x_21, 1); -lean_inc(x_24); -lean_inc(x_23); -lean_dec(x_21); -x_25 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_25, 0, x_23); -lean_ctor_set(x_25, 1, x_24); -return x_25; +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_26, 0); +x_29 = lean_ctor_get(x_26, 1); +lean_inc(x_29); +lean_inc(x_28); +lean_dec(x_26); +x_30 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +return x_30; +} } } else { -uint8_t x_26; lean_object* x_27; -x_26 = 3; -x_27 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5(x_4, x_1, x_2, x_3, x_26, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_4); -return x_27; +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_9, 1); +lean_inc(x_31); +lean_dec(x_9); +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___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); +x_37 = lean_nat_dec_eq(x_34, x_36); +lean_dec(x_36); +lean_dec(x_34); +if (x_37 == 0) +{ +lean_object* x_38; +x_38 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_38, 0, x_1); +lean_ctor_set(x_38, 1, x_31); +return x_38; +} +else +{ +lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_39 = l_Lean_Expr_appArg_x21(x_1); +lean_dec(x_1); +x_40 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getNestedProjectionArg(x_39, x_2, x_3, x_4, x_5, x_31); +x_41 = lean_ctor_get(x_40, 0); +lean_inc(x_41); +x_42 = lean_ctor_get(x_40, 1); +lean_inc(x_42); +if (lean_is_exclusive(x_40)) { + lean_ctor_release(x_40, 0); + lean_ctor_release(x_40, 1); + x_43 = x_40; +} else { + lean_dec_ref(x_40); + x_43 = lean_box(0); +} +if (lean_is_scalar(x_43)) { + x_44 = lean_alloc_ctor(0, 2, 0); +} else { + x_44 = x_43; +} +lean_ctor_set(x_44, 0, x_41); +lean_ctor_set(x_44, 1, x_42); +return x_44; +} +} } } else { -uint8_t x_28; lean_object* x_29; -lean_dec(x_13); -x_28 = 1; -x_29 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5(x_4, x_1, x_2, x_3, x_28, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_object* x_45; +lean_dec(x_7); +x_45 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_45, 0, x_1); +lean_ctor_set(x_45, 1, x_6); +return x_45; +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getNestedProjectionArg___lambda__1___boxed(lean_object* x_1, 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_Structure_0__Lean_Elab_Command_getNestedProjectionArg___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_29; +lean_dec(x_3); +lean_dec(x_2); +return x_8; } } -else +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getNestedProjectionArg___boxed(lean_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_30; lean_object* x_31; -lean_dec(x_13); -x_30 = 0; -x_31 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5(x_4, x_1, x_2, x_3, x_30, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_object* x_7; +x_7 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getNestedProjectionArg(x_1, x_2, x_3, x_4, x_5, x_6); +lean_dec(x_5); lean_dec(x_4); -return x_31; +lean_dec(x_3); +lean_dec(x_2); +return x_7; +} } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; lean_object* x_9; +x_8 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_8, 0, x_1); +x_9 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_9, 0, x_8); +lean_ctor_set(x_9, 1, x_7); +return x_9; } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__1() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("structSimpleBinder", 18, 18); +x_1 = lean_mk_string_unchecked("invalid projection name ", 24, 24); return x_1; } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__2() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__2() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__1; -x_2 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__2; -x_3 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__1; -x_4 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__1; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__3() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("(", 1, 1); -return x_1; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__4() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__4() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked(")", 1, 1); -return x_1; +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_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5(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___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -uint8_t x_14; -x_14 = lean_usize_dec_eq(x_4, x_5); -if (x_14 == 0) +lean_object* x_9; +x_9 = l_Lean_Expr_getAppFn(x_3); +if (lean_obj_tag(x_9) == 4) { -lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; lean_object* x_31; uint8_t x_32; lean_object* x_33; lean_object* x_34; -x_15 = lean_array_uget(x_3, x_4); -lean_inc(x_15); -x_16 = l_Lean_Syntax_getKind(x_15); -x_17 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__2; -x_18 = lean_name_eq(x_16, x_17); -lean_dec(x_16); -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 = lean_ctor_get_uint8(x_11, sizeof(void*)*12); -x_31 = lean_ctor_get(x_11, 11); -x_32 = lean_ctor_get_uint8(x_11, sizeof(void*)*12 + 1); -x_33 = l_Lean_replaceRef(x_15, x_24); -lean_inc(x_31); -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_34 = lean_alloc_ctor(0, 12, 2); -lean_ctor_set(x_34, 0, x_19); -lean_ctor_set(x_34, 1, x_20); -lean_ctor_set(x_34, 2, x_21); -lean_ctor_set(x_34, 3, x_22); -lean_ctor_set(x_34, 4, x_23); -lean_ctor_set(x_34, 5, x_33); -lean_ctor_set(x_34, 6, x_25); -lean_ctor_set(x_34, 7, x_26); -lean_ctor_set(x_34, 8, x_27); -lean_ctor_set(x_34, 9, x_28); -lean_ctor_set(x_34, 10, x_29); -lean_ctor_set(x_34, 11, x_31); -lean_ctor_set_uint8(x_34, sizeof(void*)*12, x_30); -lean_ctor_set_uint8(x_34, sizeof(void*)*12 + 1, x_32); -if (x_18 == 0) -{ -lean_object* x_35; lean_object* x_36; -x_35 = lean_box(0); -lean_inc(x_12); +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_9, 0); lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_2); -x_36 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6(x_6, x_2, x_1, x_15, x_35, x_7, x_8, x_9, x_10, x_34, x_12, x_13); -if (lean_obj_tag(x_36) == 0) +lean_dec(x_9); +lean_inc(x_10); +x_11 = l_Lean_getProjectionFnInfo_x3f___at_Lean_Meta_getStuckMVar_x3f___spec__1(x_10, x_4, x_5, x_6, x_7, x_8); +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +if (lean_obj_tag(x_12) == 0) { -lean_object* x_37; lean_object* x_38; size_t x_39; size_t x_40; -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 = 1; -x_40 = lean_usize_add(x_4, x_39); -x_4 = x_40; -x_6 = x_37; -x_13 = x_38; -goto _start; +lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_dec(x_10); +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +x_14 = lean_box(0); +x_15 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__1(x_3, x_14, x_4, x_5, x_6, x_7, x_13); +return x_15; } else { -uint8_t x_42; +lean_object* x_16; +x_16 = lean_ctor_get(x_12, 0); +lean_inc(x_16); lean_dec(x_12); +if (lean_obj_tag(x_10) == 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_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_17 = lean_ctor_get(x_11, 1); +lean_inc(x_17); +lean_dec(x_11); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +x_19 = lean_ctor_get(x_10, 1); +lean_inc(x_19); lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_2); -x_42 = !lean_is_exclusive(x_36); -if (x_42 == 0) +x_20 = lean_unsigned_to_nat(0u); +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__4; +lean_inc(x_21); +x_23 = lean_mk_array(x_21, x_22); +x_24 = lean_unsigned_to_nat(1u); +x_25 = lean_nat_sub(x_21, x_24); +lean_dec(x_21); +lean_inc(x_3); +x_26 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_3, x_23, x_25); +x_27 = l_Array_get_x3f___rarg(x_26, x_18); +if (lean_obj_tag(x_27) == 0) { -return x_36; +lean_object* x_28; lean_object* x_29; +lean_dec(x_26); +lean_dec(x_19); +lean_dec(x_18); +x_28 = lean_box(0); +x_29 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__1(x_3, x_28, x_4, x_5, x_6, x_7, x_17); +return x_29; } else { -lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_43 = lean_ctor_get(x_36, 0); -x_44 = lean_ctor_get(x_36, 1); -lean_inc(x_44); -lean_inc(x_43); -lean_dec(x_36); -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_30; lean_object* x_31; uint8_t x_32; +x_30 = lean_ctor_get(x_27, 0); +lean_inc(x_30); +lean_dec(x_27); +x_31 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getNestedProjectionArg(x_30, x_4, x_5, x_6, x_7, x_17); +x_32 = !lean_is_exclusive(x_31); +if (x_32 == 0) { -lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; -x_46 = lean_unsigned_to_nat(0u); -x_47 = l_Lean_Syntax_getArg(x_15, x_46); -x_48 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__3; -x_49 = 0; -x_50 = l_Lean_mkAtomFrom(x_15, x_48, x_49); -x_51 = lean_unsigned_to_nat(1u); -x_52 = l_Lean_Syntax_getArg(x_15, x_51); -x_53 = lean_box(0); -x_54 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_54, 0, x_52); -lean_ctor_set(x_54, 1, x_53); -x_55 = lean_array_mk(x_54); -x_56 = lean_box(2); -x_57 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__6; -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_unsigned_to_nat(2u); -x_60 = l_Lean_Syntax_getArg(x_15, x_59); -x_61 = lean_unsigned_to_nat(3u); -x_62 = l_Lean_Syntax_getArg(x_15, x_61); -x_63 = lean_unsigned_to_nat(4u); -x_64 = l_Lean_Syntax_getArg(x_15, x_63); -x_65 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__4; -x_66 = l_Lean_mkAtomFrom(x_15, x_65, x_49); -lean_dec(x_15); -x_67 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_67, 0, x_66); -lean_ctor_set(x_67, 1, x_53); -x_68 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_68, 0, x_64); -lean_ctor_set(x_68, 1, x_67); -x_69 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_69, 0, x_62); -lean_ctor_set(x_69, 1, x_68); -x_70 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_70, 0, x_60); -lean_ctor_set(x_70, 1, x_69); -x_71 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_71, 0, x_58); -lean_ctor_set(x_71, 1, x_70); -x_72 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_72, 0, x_50); -lean_ctor_set(x_72, 1, x_71); -x_73 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_73, 0, x_47); -lean_ctor_set(x_73, 1, x_72); -x_74 = lean_array_mk(x_73); -x_75 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__2; -x_76 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_76, 0, x_56); -lean_ctor_set(x_76, 1, x_75); -lean_ctor_set(x_76, 2, x_74); -x_77 = lean_box(0); -lean_inc(x_12); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_2); -x_78 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6(x_6, x_2, x_1, x_76, x_77, x_7, x_8, x_9, x_10, x_34, x_12, x_13); -if (lean_obj_tag(x_78) == 0) +lean_object* x_33; lean_object* x_34; uint8_t x_35; +x_33 = lean_ctor_get(x_31, 0); +x_34 = lean_ctor_get(x_31, 1); +x_35 = lean_expr_eqv(x_33, x_1); +lean_dec(x_33); +if (x_35 == 0) { -lean_object* x_79; lean_object* x_80; size_t x_81; size_t x_82; -x_79 = lean_ctor_get(x_78, 0); -lean_inc(x_79); -x_80 = lean_ctor_get(x_78, 1); -lean_inc(x_80); -lean_dec(x_78); -x_81 = 1; -x_82 = lean_usize_add(x_4, x_81); -x_4 = x_82; -x_6 = x_79; -x_13 = x_80; -goto _start; +lean_object* x_36; lean_object* x_37; +lean_free_object(x_31); +lean_dec(x_26); +lean_dec(x_19); +lean_dec(x_18); +x_36 = lean_box(0); +x_37 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__1(x_3, x_36, x_4, x_5, x_6, x_7, x_34); +return x_37; } else { -uint8_t x_84; -lean_dec(x_12); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_2); -x_84 = !lean_is_exclusive(x_78); -if (x_84 == 0) +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_box(0); +x_39 = l_Lean_Name_str___override(x_38, x_19); +x_40 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f(x_2, x_39); +lean_dec(x_39); +if (lean_obj_tag(x_40) == 0) { -return x_78; +lean_object* x_41; lean_object* x_42; +lean_free_object(x_31); +lean_dec(x_26); +lean_dec(x_18); +x_41 = lean_box(0); +x_42 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__1(x_3, x_41, x_4, x_5, x_6, x_7, x_34); +return x_42; } else { -lean_object* x_85; lean_object* x_86; lean_object* x_87; -x_85 = lean_ctor_get(x_78, 0); -x_86 = lean_ctor_get(x_78, 1); -lean_inc(x_86); -lean_inc(x_85); -lean_dec(x_78); -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; -} -} -} +uint8_t x_43; +lean_dec(x_3); +x_43 = !lean_is_exclusive(x_40); +if (x_43 == 0) +{ +lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_44 = lean_ctor_get(x_40, 0); +x_45 = lean_ctor_get(x_44, 3); +lean_inc(x_45); +lean_dec(x_44); +x_46 = lean_nat_add(x_18, x_24); +lean_dec(x_18); +x_47 = lean_array_get_size(x_26); +x_48 = l_Array_toSubarray___rarg(x_26, x_46, x_47); +x_49 = l_Array_ofSubarray___rarg(x_48); +lean_dec(x_48); +x_50 = l_Lean_mkAppN(x_45, x_49); +lean_dec(x_49); +lean_ctor_set_tag(x_40, 0); +lean_ctor_set(x_40, 0, x_50); +lean_ctor_set(x_31, 0, x_40); +return x_31; } else { -lean_object* x_88; -lean_dec(x_12); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_2); -x_88 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_88, 0, x_6); -lean_ctor_set(x_88, 1, x_13); -return x_88; +lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; +x_51 = lean_ctor_get(x_40, 0); +lean_inc(x_51); +lean_dec(x_40); +x_52 = lean_ctor_get(x_51, 3); +lean_inc(x_52); +lean_dec(x_51); +x_53 = lean_nat_add(x_18, x_24); +lean_dec(x_18); +x_54 = lean_array_get_size(x_26); +x_55 = l_Array_toSubarray___rarg(x_26, x_53, x_54); +x_56 = l_Array_ofSubarray___rarg(x_55); +lean_dec(x_55); +x_57 = l_Lean_mkAppN(x_52, x_56); +lean_dec(x_56); +x_58 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_58, 0, x_57); +lean_ctor_set(x_31, 0, x_58); +return x_31; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___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: -{ -uint8_t x_14; -x_14 = lean_usize_dec_eq(x_4, x_5); -if (x_14 == 0) -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; lean_object* x_31; uint8_t x_32; lean_object* x_33; lean_object* x_34; -x_15 = lean_array_uget(x_3, x_4); -lean_inc(x_15); -x_16 = l_Lean_Syntax_getKind(x_15); -x_17 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__2; -x_18 = lean_name_eq(x_16, x_17); -lean_dec(x_16); -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 = lean_ctor_get_uint8(x_11, sizeof(void*)*12); -x_31 = lean_ctor_get(x_11, 11); -x_32 = lean_ctor_get_uint8(x_11, sizeof(void*)*12 + 1); -x_33 = l_Lean_replaceRef(x_15, x_24); -lean_inc(x_31); -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_34 = lean_alloc_ctor(0, 12, 2); -lean_ctor_set(x_34, 0, x_19); -lean_ctor_set(x_34, 1, x_20); -lean_ctor_set(x_34, 2, x_21); -lean_ctor_set(x_34, 3, x_22); -lean_ctor_set(x_34, 4, x_23); -lean_ctor_set(x_34, 5, x_33); -lean_ctor_set(x_34, 6, x_25); -lean_ctor_set(x_34, 7, x_26); -lean_ctor_set(x_34, 8, x_27); -lean_ctor_set(x_34, 9, x_28); -lean_ctor_set(x_34, 10, x_29); -lean_ctor_set(x_34, 11, x_31); -lean_ctor_set_uint8(x_34, sizeof(void*)*12, x_30); -lean_ctor_set_uint8(x_34, sizeof(void*)*12 + 1, x_32); -if (x_18 == 0) +} +else { -lean_object* x_35; lean_object* x_36; -x_35 = lean_box(0); -lean_inc(x_12); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_2); -x_36 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6(x_6, x_2, x_1, x_15, x_35, x_7, x_8, x_9, x_10, x_34, x_12, x_13); -if (lean_obj_tag(x_36) == 0) +lean_object* x_59; lean_object* x_60; uint8_t x_61; +x_59 = lean_ctor_get(x_31, 0); +x_60 = lean_ctor_get(x_31, 1); +lean_inc(x_60); +lean_inc(x_59); +lean_dec(x_31); +x_61 = lean_expr_eqv(x_59, x_1); +lean_dec(x_59); +if (x_61 == 0) { -lean_object* x_37; lean_object* x_38; size_t x_39; size_t x_40; -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 = 1; -x_40 = lean_usize_add(x_4, x_39); -x_4 = x_40; -x_6 = x_37; -x_13 = x_38; -goto _start; +lean_object* x_62; lean_object* x_63; +lean_dec(x_26); +lean_dec(x_19); +lean_dec(x_18); +x_62 = lean_box(0); +x_63 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__1(x_3, x_62, x_4, x_5, x_6, x_7, x_60); +return x_63; } else { -uint8_t x_42; -lean_dec(x_12); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_2); -x_42 = !lean_is_exclusive(x_36); -if (x_42 == 0) +lean_object* x_64; lean_object* x_65; lean_object* x_66; +x_64 = lean_box(0); +x_65 = l_Lean_Name_str___override(x_64, x_19); +x_66 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f(x_2, x_65); +lean_dec(x_65); +if (lean_obj_tag(x_66) == 0) { -return x_36; +lean_object* x_67; lean_object* x_68; +lean_dec(x_26); +lean_dec(x_18); +x_67 = lean_box(0); +x_68 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__1(x_3, x_67, x_4, x_5, x_6, x_7, x_60); +return x_68; } else { -lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_43 = lean_ctor_get(x_36, 0); -x_44 = lean_ctor_get(x_36, 1); -lean_inc(x_44); -lean_inc(x_43); -lean_dec(x_36); -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_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_dec(x_3); +x_69 = lean_ctor_get(x_66, 0); +lean_inc(x_69); +if (lean_is_exclusive(x_66)) { + lean_ctor_release(x_66, 0); + x_70 = x_66; +} else { + lean_dec_ref(x_66); + x_70 = lean_box(0); +} +x_71 = lean_ctor_get(x_69, 3); +lean_inc(x_71); +lean_dec(x_69); +x_72 = lean_nat_add(x_18, x_24); +lean_dec(x_18); +x_73 = lean_array_get_size(x_26); +x_74 = l_Array_toSubarray___rarg(x_26, x_72, x_73); +x_75 = l_Array_ofSubarray___rarg(x_74); +lean_dec(x_74); +x_76 = l_Lean_mkAppN(x_71, x_75); +lean_dec(x_75); +if (lean_is_scalar(x_70)) { + x_77 = lean_alloc_ctor(0, 1, 0); +} else { + x_77 = x_70; + lean_ctor_set_tag(x_77, 0); +} +lean_ctor_set(x_77, 0, x_76); +x_78 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_78, 0, x_77); +lean_ctor_set(x_78, 1, x_60); +return x_78; +} +} } } } else { -lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; -x_46 = lean_unsigned_to_nat(0u); -x_47 = l_Lean_Syntax_getArg(x_15, x_46); -x_48 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__3; -x_49 = 0; -x_50 = l_Lean_mkAtomFrom(x_15, x_48, x_49); -x_51 = lean_unsigned_to_nat(1u); -x_52 = l_Lean_Syntax_getArg(x_15, x_51); -x_53 = lean_box(0); -x_54 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_54, 0, x_52); -lean_ctor_set(x_54, 1, x_53); -x_55 = lean_array_mk(x_54); -x_56 = lean_box(2); -x_57 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__6; -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_unsigned_to_nat(2u); -x_60 = l_Lean_Syntax_getArg(x_15, x_59); -x_61 = lean_unsigned_to_nat(3u); -x_62 = l_Lean_Syntax_getArg(x_15, x_61); -x_63 = lean_unsigned_to_nat(4u); -x_64 = l_Lean_Syntax_getArg(x_15, x_63); -x_65 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__4; -x_66 = l_Lean_mkAtomFrom(x_15, x_65, x_49); -lean_dec(x_15); -x_67 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_67, 0, x_66); -lean_ctor_set(x_67, 1, x_53); -x_68 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_68, 0, x_64); -lean_ctor_set(x_68, 1, x_67); -x_69 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_69, 0, x_62); -lean_ctor_set(x_69, 1, x_68); -x_70 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_70, 0, x_60); -lean_ctor_set(x_70, 1, x_69); -x_71 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_71, 0, x_58); -lean_ctor_set(x_71, 1, x_70); -x_72 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_72, 0, x_50); -lean_ctor_set(x_72, 1, x_71); -x_73 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_73, 0, x_47); -lean_ctor_set(x_73, 1, x_72); -x_74 = lean_array_mk(x_73); -x_75 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__2; -x_76 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_76, 0, x_56); -lean_ctor_set(x_76, 1, x_75); -lean_ctor_set(x_76, 2, x_74); -x_77 = lean_box(0); -lean_inc(x_12); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_2); -x_78 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6(x_6, x_2, x_1, x_76, x_77, x_7, x_8, x_9, x_10, x_34, x_12, x_13); -if (lean_obj_tag(x_78) == 0) -{ -lean_object* x_79; lean_object* x_80; size_t x_81; size_t x_82; -x_79 = lean_ctor_get(x_78, 0); -lean_inc(x_79); -x_80 = lean_ctor_get(x_78, 1); -lean_inc(x_80); -lean_dec(x_78); -x_81 = 1; -x_82 = lean_usize_add(x_4, x_81); -x_4 = x_82; -x_6 = x_79; -x_13 = x_80; -goto _start; -} -else +uint8_t x_79; +lean_dec(x_16); +lean_dec(x_3); +x_79 = !lean_is_exclusive(x_11); +if (x_79 == 0) { -uint8_t x_84; -lean_dec(x_12); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_2); -x_84 = !lean_is_exclusive(x_78); -if (x_84 == 0) +lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; uint8_t x_87; +x_80 = lean_ctor_get(x_11, 1); +x_81 = lean_ctor_get(x_11, 0); +lean_dec(x_81); +x_82 = l_Lean_MessageData_ofName(x_10); +x_83 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__2; +lean_ctor_set_tag(x_11, 7); +lean_ctor_set(x_11, 1, x_82); +lean_ctor_set(x_11, 0, x_83); +x_84 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3; +x_85 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_85, 0, x_11); +lean_ctor_set(x_85, 1, x_84); +x_86 = l_Lean_throwError___at_Lean_Meta_mkSimpCongrTheorem___spec__4(x_85, x_4, x_5, x_6, x_7, x_80); +x_87 = !lean_is_exclusive(x_86); +if (x_87 == 0) { -return x_78; +return x_86; } else { -lean_object* x_85; lean_object* x_86; lean_object* x_87; -x_85 = lean_ctor_get(x_78, 0); -x_86 = lean_ctor_get(x_78, 1); -lean_inc(x_86); -lean_inc(x_85); -lean_dec(x_78); -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_88; lean_object* x_89; lean_object* x_90; +x_88 = lean_ctor_get(x_86, 0); +x_89 = lean_ctor_get(x_86, 1); +lean_inc(x_89); +lean_inc(x_88); +lean_dec(x_86); +x_90 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_90, 0, x_88); +lean_ctor_set(x_90, 1, x_89); +return x_90; } } else { -lean_object* x_88; -lean_dec(x_12); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_2); -x_88 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_88, 0, x_6); -lean_ctor_set(x_88, 1, x_13); -return x_88; -} +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_11, 1); +lean_inc(x_91); +lean_dec(x_11); +x_92 = l_Lean_MessageData_ofName(x_10); +x_93 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__2; +x_94 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_94, 0, x_93); +lean_ctor_set(x_94, 1, x_92); +x_95 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3; +x_96 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_96, 0, x_94); +lean_ctor_set(x_96, 1, x_95); +x_97 = l_Lean_throwError___at_Lean_Meta_mkSimpCongrTheorem___spec__4(x_96, x_4, x_5, x_6, x_7, x_91); +x_98 = lean_ctor_get(x_97, 0); +lean_inc(x_98); +x_99 = lean_ctor_get(x_97, 1); +lean_inc(x_99); +if (lean_is_exclusive(x_97)) { + lean_ctor_release(x_97, 0); + lean_ctor_release(x_97, 1); + x_100 = x_97; +} else { + lean_dec_ref(x_97); + x_100 = lean_box(0); } +if (lean_is_scalar(x_100)) { + x_101 = lean_alloc_ctor(1, 2, 0); +} else { + x_101 = x_100; } -static lean_object* _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("note: this linter can be disabled with `set_option ", 51, 51); -return x_1; +lean_ctor_set(x_101, 0, x_98); +lean_ctor_set(x_101, 1, x_99); +return x_101; } } -static lean_object* _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; } } -static lean_object* _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__3() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked(" false`", 7, 7); -return x_1; +lean_object* x_102; lean_object* x_103; +lean_dec(x_9); +x_102 = lean_box(0); +x_103 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__1(x_3, x_102, x_4, x_5, x_6, x_7, x_8); +return x_103; +} } } -static lean_object* _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__4() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__3___closed__1() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__3; -x_2 = l_Lean_stringToMessageData(x_1); +x_1 = lean_box(0); +x_2 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__5() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("\n", 1, 1); -return x_1; -} -} -static lean_object* _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__6() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___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_1; lean_object* x_2; -x_1 = l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__5; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +lean_object* x_7; lean_object* x_8; +x_7 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__3___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); +return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___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___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -uint8_t x_11; -x_11 = !lean_is_exclusive(x_1); +lean_object* x_10; uint8_t x_11; +x_10 = lean_st_ref_get(x_8, x_9); +x_11 = !lean_is_exclusive(x_10); if (x_11 == 0) { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; 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; -x_12 = lean_ctor_get(x_1, 0); -x_13 = lean_ctor_get(x_1, 1); -lean_dec(x_13); -lean_inc(x_12); -x_14 = l_Lean_MessageData_ofName(x_12); -x_15 = l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__2; -lean_ctor_set_tag(x_1, 7); -lean_ctor_set(x_1, 1, x_14); -lean_ctor_set(x_1, 0, x_15); -x_16 = l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__4; -x_17 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_17, 0, x_1); -lean_ctor_set(x_17, 1, x_16); -x_18 = l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__4; -x_19 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_19, 0, x_18); -lean_ctor_set(x_19, 1, x_3); -x_20 = l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__6; -x_21 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_21, 0, x_19); -lean_ctor_set(x_21, 1, x_20); -x_22 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_22, 0, x_21); -lean_ctor_set(x_22, 1, x_17); -x_23 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_23, 0, x_22); -lean_ctor_set(x_23, 1, x_18); -x_24 = lean_alloc_ctor(8, 2, 0); -lean_ctor_set(x_24, 0, x_12); -lean_ctor_set(x_24, 1, x_23); -x_25 = 1; -x_26 = l_Lean_logAt___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__2(x_2, x_24, x_25, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_26; -} -else +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_12 = lean_ctor_get(x_10, 0); +x_13 = lean_ctor_get(x_10, 1); +x_14 = lean_ctor_get(x_12, 0); +lean_inc(x_14); +lean_dec(x_12); +x_15 = l_Lean_Meta_getStructureName(x_1, x_5, x_6, x_7, x_8, x_13); +if (lean_obj_tag(x_15) == 0) { -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; lean_object* x_41; -x_27 = lean_ctor_get(x_1, 0); -lean_inc(x_27); -lean_dec(x_1); -lean_inc(x_27); -x_28 = l_Lean_MessageData_ofName(x_27); -x_29 = l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__2; -x_30 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_30, 0, x_29); -lean_ctor_set(x_30, 1, x_28); -x_31 = l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__4; -x_32 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_32, 0, x_30); -lean_ctor_set(x_32, 1, x_31); -x_33 = l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__4; -x_34 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_34, 0, x_33); -lean_ctor_set(x_34, 1, x_3); -x_35 = l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__6; -x_36 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_36, 0, x_34); -lean_ctor_set(x_36, 1, x_35); -x_37 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_37, 0, x_36); -lean_ctor_set(x_37, 1, x_32); -x_38 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_38, 0, x_37); -lean_ctor_set(x_38, 1, x_33); -x_39 = lean_alloc_ctor(8, 2, 0); -lean_ctor_set(x_39, 0, x_27); -lean_ctor_set(x_39, 1, x_38); -x_40 = 1; -x_41 = l_Lean_logAt___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__2(x_2, x_39, x_40, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_41; -} -} -} -LEAN_EXPORT lean_object* l_Lean_Linter_logLintIf___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___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: +uint8_t x_16; +x_16 = !lean_is_exclusive(x_15); +if (x_16 == 0) { -lean_object* x_11; uint8_t x_12; -x_11 = lean_ctor_get(x_8, 2); -lean_inc(x_11); -lean_inc(x_1); -x_12 = l_Lean_Linter_getLinterValue(x_1, x_11); -lean_dec(x_11); -if (x_12 == 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); +x_19 = l_Lean_getFieldInfo_x3f(x_14, x_17, x_3); +lean_dec(x_14); +if (lean_obj_tag(x_19) == 0) { -lean_object* x_13; lean_object* x_14; +lean_free_object(x_10); lean_dec(x_8); -lean_dec(x_3); -lean_dec(x_1); -x_13 = lean_box(0); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_13); -lean_ctor_set(x_14, 1, x_10); -return x_14; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_ctor_set(x_15, 0, x_2); +return x_15; } else { -lean_object* x_15; -x_15 = l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_object* x_20; lean_object* x_21; +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +lean_dec(x_19); +x_21 = lean_ctor_get(x_20, 3); +lean_inc(x_21); +lean_dec(x_20); +if (lean_obj_tag(x_21) == 0) +{ +lean_free_object(x_10); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_ctor_set(x_15, 0, x_2); return x_15; } +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_free_object(x_15); +x_22 = lean_ctor_get(x_21, 0); +lean_inc(x_22); +lean_dec(x_21); +x_23 = lean_box(0); +lean_ctor_set_tag(x_10, 1); +lean_ctor_set(x_10, 1, x_23); +lean_ctor_set(x_10, 0, x_22); +x_24 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_24, 0, x_2); +lean_ctor_set(x_24, 1, x_10); +x_25 = lean_array_mk(x_24); +x_26 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__15; +x_27 = l_Lean_Meta_mkAppM(x_26, x_25, x_5, x_6, x_7, x_8, x_18); +if (lean_obj_tag(x_27) == 0) +{ +uint8_t x_28; +x_28 = !lean_is_exclusive(x_27); +if (x_28 == 0) +{ +return x_27; } -} -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__1() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; -x_2 = lean_array_get_size(x_1); -return x_2; +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_27, 0); +x_30 = lean_ctor_get(x_27, 1); +lean_inc(x_30); +lean_inc(x_29); +lean_dec(x_27); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_29); +lean_ctor_set(x_31, 1, x_30); +return x_31; } } -static uint8_t _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__2() { -_start: +else { -lean_object* x_1; lean_object* x_2; uint8_t x_3; -x_1 = lean_unsigned_to_nat(0u); -x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__1; -x_3 = lean_nat_dec_lt(x_1, x_2); -return x_3; -} +uint8_t x_32; +x_32 = !lean_is_exclusive(x_27); +if (x_32 == 0) +{ +return x_27; } -static uint8_t _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__3() { -_start: +else { -lean_object* x_1; uint8_t x_2; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__1; -x_2 = lean_nat_dec_le(x_1, x_1); -return x_2; +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_27, 0); +x_34 = lean_ctor_get(x_27, 1); +lean_inc(x_34); +lean_inc(x_33); +lean_dec(x_27); +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +return x_35; } } -static size_t _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__4() { -_start: -{ -lean_object* x_1; size_t x_2; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__1; -x_2 = lean_usize_of_nat(x_1); -return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -lean_object* x_12; lean_object* x_13; uint8_t x_14; -x_12 = lean_unsigned_to_nat(5u); -x_13 = l_Lean_Syntax_getArg(x_1, x_12); -x_14 = l_Lean_Syntax_isNone(x_13); -if (x_14 == 0) +} +else { -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; -x_15 = lean_unsigned_to_nat(2u); -x_16 = l_Lean_Syntax_getArg(x_13, x_15); -lean_dec(x_13); -x_17 = lean_unsigned_to_nat(0u); -x_18 = l_Lean_Syntax_getArg(x_16, x_17); -lean_dec(x_16); -x_19 = l_Lean_Syntax_getArgs(x_18); -lean_dec(x_18); -x_20 = lean_array_get_size(x_19); -x_21 = lean_nat_dec_lt(x_17, x_20); -if (x_21 == 0) +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_15, 0); +x_37 = lean_ctor_get(x_15, 1); +lean_inc(x_37); +lean_inc(x_36); +lean_dec(x_15); +x_38 = l_Lean_getFieldInfo_x3f(x_14, x_36, x_3); +lean_dec(x_14); +if (lean_obj_tag(x_38) == 0) { -lean_object* x_22; lean_object* x_23; -lean_dec(x_20); -lean_dec(x_19); -lean_dec(x_10); +lean_object* x_39; +lean_free_object(x_10); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_3); -x_22 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; -x_23 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_23, 0, x_22); -lean_ctor_set(x_23, 1, x_11); -return x_23; +x_39 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_39, 0, x_2); +lean_ctor_set(x_39, 1, x_37); +return x_39; } else { -uint8_t x_24; -x_24 = lean_nat_dec_le(x_20, x_20); -if (x_24 == 0) +lean_object* x_40; lean_object* x_41; +x_40 = lean_ctor_get(x_38, 0); +lean_inc(x_40); +lean_dec(x_38); +x_41 = lean_ctor_get(x_40, 3); +lean_inc(x_41); +lean_dec(x_40); +if (lean_obj_tag(x_41) == 0) { -lean_object* x_25; lean_object* x_26; -lean_dec(x_20); -lean_dec(x_19); -lean_dec(x_10); +lean_object* x_42; +lean_free_object(x_10); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_3); -x_25 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___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_11); -return x_26; +x_42 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_42, 0, x_2); +lean_ctor_set(x_42, 1, x_37); +return x_42; } else { -size_t x_27; size_t x_28; lean_object* x_29; lean_object* x_30; -x_27 = 0; -x_28 = lean_usize_of_nat(x_20); -lean_dec(x_20); -x_29 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; -x_30 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5(x_2, x_3, x_19, x_27, x_28, x_29, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_19); -return x_30; +lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_43 = lean_ctor_get(x_41, 0); +lean_inc(x_43); +lean_dec(x_41); +x_44 = lean_box(0); +lean_ctor_set_tag(x_10, 1); +lean_ctor_set(x_10, 1, x_44); +lean_ctor_set(x_10, 0, x_43); +x_45 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_45, 0, x_2); +lean_ctor_set(x_45, 1, x_10); +x_46 = lean_array_mk(x_45); +x_47 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__15; +x_48 = l_Lean_Meta_mkAppM(x_47, x_46, x_5, x_6, x_7, x_8, x_37); +if (lean_obj_tag(x_48) == 0) +{ +lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_49 = lean_ctor_get(x_48, 0); +lean_inc(x_49); +x_50 = lean_ctor_get(x_48, 1); +lean_inc(x_50); +if (lean_is_exclusive(x_48)) { + lean_ctor_release(x_48, 0); + lean_ctor_release(x_48, 1); + x_51 = x_48; +} else { + lean_dec_ref(x_48); + x_51 = lean_box(0); } +if (lean_is_scalar(x_51)) { + x_52 = lean_alloc_ctor(0, 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; } else { -uint8_t x_31; -lean_dec(x_13); -x_31 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__2; -if (x_31 == 0) +lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; +x_53 = lean_ctor_get(x_48, 0); +lean_inc(x_53); +x_54 = lean_ctor_get(x_48, 1); +lean_inc(x_54); +if (lean_is_exclusive(x_48)) { + lean_ctor_release(x_48, 0); + lean_ctor_release(x_48, 1); + x_55 = x_48; +} else { + lean_dec_ref(x_48); + x_55 = lean_box(0); +} +if (lean_is_scalar(x_55)) { + x_56 = lean_alloc_ctor(1, 2, 0); +} else { + x_56 = x_55; +} +lean_ctor_set(x_56, 0, x_53); +lean_ctor_set(x_56, 1, x_54); +return x_56; +} +} +} +} +} +else { -lean_object* x_32; lean_object* x_33; -lean_dec(x_10); +uint8_t x_57; +lean_dec(x_14); +lean_free_object(x_10); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); -x_32 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___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_11); -return x_33; +lean_dec(x_2); +x_57 = !lean_is_exclusive(x_15); +if (x_57 == 0) +{ +return x_15; } else { -uint8_t x_34; -x_34 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__3; -if (x_34 == 0) -{ -lean_object* x_35; lean_object* x_36; -lean_dec(x_10); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -x_35 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; -x_36 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_36, 0, x_35); -lean_ctor_set(x_36, 1, x_11); -return x_36; +lean_object* x_58; lean_object* x_59; lean_object* x_60; +x_58 = lean_ctor_get(x_15, 0); +x_59 = lean_ctor_get(x_15, 1); +lean_inc(x_59); +lean_inc(x_58); +lean_dec(x_15); +x_60 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_60, 0, x_58); +lean_ctor_set(x_60, 1, x_59); +return x_60; +} +} } else { -size_t x_37; lean_object* x_38; size_t x_39; lean_object* x_40; -x_37 = 0; -x_38 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; -x_39 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__4; -x_40 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__6(x_2, x_3, x_38, x_37, x_39, x_38, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -return x_40; +lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; +x_61 = lean_ctor_get(x_10, 0); +x_62 = lean_ctor_get(x_10, 1); +lean_inc(x_62); +lean_inc(x_61); +lean_dec(x_10); +x_63 = lean_ctor_get(x_61, 0); +lean_inc(x_63); +lean_dec(x_61); +x_64 = l_Lean_Meta_getStructureName(x_1, x_5, x_6, x_7, x_8, x_62); +if (lean_obj_tag(x_64) == 0) +{ +lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; +x_65 = lean_ctor_get(x_64, 0); +lean_inc(x_65); +x_66 = lean_ctor_get(x_64, 1); +lean_inc(x_66); +if (lean_is_exclusive(x_64)) { + lean_ctor_release(x_64, 0); + lean_ctor_release(x_64, 1); + x_67 = x_64; +} else { + lean_dec_ref(x_64); + x_67 = lean_box(0); } +x_68 = l_Lean_getFieldInfo_x3f(x_63, x_65, x_3); +lean_dec(x_63); +if (lean_obj_tag(x_68) == 0) +{ +lean_object* x_69; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +if (lean_is_scalar(x_67)) { + x_69 = lean_alloc_ctor(0, 2, 0); +} else { + x_69 = x_67; } +lean_ctor_set(x_69, 0, x_2); +lean_ctor_set(x_69, 1, x_66); +return x_69; } +else +{ +lean_object* x_70; lean_object* x_71; +x_70 = lean_ctor_get(x_68, 0); +lean_inc(x_70); +lean_dec(x_68); +x_71 = lean_ctor_get(x_70, 3); +lean_inc(x_71); +lean_dec(x_70); +if (lean_obj_tag(x_71) == 0) +{ +lean_object* x_72; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +if (lean_is_scalar(x_67)) { + x_72 = lean_alloc_ctor(0, 2, 0); +} else { + x_72 = x_67; } +lean_ctor_set(x_72, 0, x_2); +lean_ctor_set(x_72, 1, x_66); +return x_72; } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked(":=", 2, 2); -return x_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_dec(x_67); +x_73 = lean_ctor_get(x_71, 0); +lean_inc(x_73); +lean_dec(x_71); +x_74 = lean_box(0); +x_75 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_75, 0, x_73); +lean_ctor_set(x_75, 1, x_74); +x_76 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_76, 0, x_2); +lean_ctor_set(x_76, 1, x_75); +x_77 = lean_array_mk(x_76); +x_78 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__15; +x_79 = l_Lean_Meta_mkAppM(x_78, x_77, x_5, x_6, x_7, x_8, x_66); +if (lean_obj_tag(x_79) == 0) +{ +lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; +x_80 = lean_ctor_get(x_79, 0); +lean_inc(x_80); +x_81 = lean_ctor_get(x_79, 1); +lean_inc(x_81); +if (lean_is_exclusive(x_79)) { + lean_ctor_release(x_79, 0); + lean_ctor_release(x_79, 1); + x_82 = x_79; +} else { + lean_dec_ref(x_79); + x_82 = lean_box(0); } +if (lean_is_scalar(x_82)) { + x_83 = lean_alloc_ctor(0, 2, 0); +} else { + x_83 = x_82; } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__2() { -_start: +lean_ctor_set(x_83, 0, x_80); +lean_ctor_set(x_83, 1, x_81); +return x_83; +} +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("classTk", 7, 7); -return x_1; +lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; +x_84 = lean_ctor_get(x_79, 0); +lean_inc(x_84); +x_85 = lean_ctor_get(x_79, 1); +lean_inc(x_85); +if (lean_is_exclusive(x_79)) { + lean_ctor_release(x_79, 0); + lean_ctor_release(x_79, 1); + x_86 = x_79; +} else { + lean_dec_ref(x_79); + x_86 = lean_box(0); } +if (lean_is_scalar(x_86)) { + x_87 = lean_alloc_ctor(1, 2, 0); +} else { + x_87 = x_86; } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__1; -x_2 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__2; -x_3 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__1; -x_4 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__2; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; +lean_ctor_set(x_87, 0, x_84); +lean_ctor_set(x_87, 1, x_85); +return x_87; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("structure", 9, 9); -return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__5() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__3; -x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__4; -x_3 = lean_string_append(x_1, x_2); -return x_3; +lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; +lean_dec(x_63); +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_88 = lean_ctor_get(x_64, 0); +lean_inc(x_88); +x_89 = lean_ctor_get(x_64, 1); +lean_inc(x_89); +if (lean_is_exclusive(x_64)) { + lean_ctor_release(x_64, 0); + lean_ctor_release(x_64, 1); + x_90 = x_64; +} else { + lean_dec_ref(x_64); + x_90 = lean_box(0); } +if (lean_is_scalar(x_90)) { + x_91 = lean_alloc_ctor(1, 2, 0); +} else { + x_91 = x_90; } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__6() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked(" ... :=' has been deprecated in favor of '", 42, 42); -return x_1; +lean_ctor_set(x_91, 0, x_88); +lean_ctor_set(x_91, 1, x_89); +return x_91; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__7() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__5; -x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__6; -x_3 = lean_string_append(x_1, x_2); -return x_3; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__8() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___closed__1() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__7; -x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__4; -x_3 = lean_string_append(x_1, x_2); -return x_3; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__3___boxed), 6, 0); +return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__9() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___closed__2() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked(" ... where'.", 12, 12); +x_1 = lean_mk_string_unchecked("unsupported dependent field in ", 31, 31); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__10() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___closed__3() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__8; -x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__9; -x_3 = lean_string_append(x_1, x_2); -return x_3; +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___closed__2; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__11() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___closed__4() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__10; -x_2 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" : ", 3, 3); +return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__12() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___closed__5() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__11; -x_2 = l_Lean_MessageData_ofFormat(x_1); +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___closed__4; +x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__13() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_1; -x_1 = l_Lean_Linter_linter_deprecated; -return x_1; +lean_object* x_10; +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_1); +lean_inc(x_4); +x_10 = l_Lean_Meta_mkProjection(x_4, x_1, 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); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_13 = lean_infer_type(x_11, x_5, x_6, x_7, x_8, x_12); +if (lean_obj_tag(x_13) == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_13, 1); +lean_inc(x_15); +lean_dec(x_13); +lean_inc(x_4); +x_16 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___boxed), 8, 2); +lean_closure_set(x_16, 0, x_4); +lean_closure_set(x_16, 1, x_2); +x_17 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___closed__1; +x_18 = 0; +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_19 = l_Lean_Meta_transform___at_Lean_Meta_zetaReduce___spec__1(x_14, x_17, x_16, x_18, x_18, x_5, x_6, x_7, x_8, x_15); +if (lean_obj_tag(x_19) == 0) +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_20 = lean_ctor_get(x_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_Expr_fvarId_x21(x_4); +lean_dec(x_4); +x_23 = l_Lean_Expr_hasAnyFVar_visit___at_Lean_Expr_containsFVar___spec__1(x_22, x_20); +lean_dec(x_22); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; +x_24 = lean_box(0); +x_25 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__4(x_3, x_20, x_1, x_24, x_5, x_6, x_7, x_8, x_21); +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_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; +x_26 = l_Lean_MessageData_ofName(x_1); +x_27 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___closed__3; +x_28 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_26); +x_29 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___closed__5; +x_30 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +x_31 = l_Lean_MessageData_ofExpr(x_20); +x_32 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_31); +x_33 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3; +x_34 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_34, 0, x_32); +lean_ctor_set(x_34, 1, x_33); +x_35 = l_Lean_throwError___at_Lean_Meta_mkSimpCongrTheorem___spec__4(x_34, x_5, x_6, x_7, x_8, x_21); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_36 = !lean_is_exclusive(x_35); +if (x_36 == 0) +{ +return x_35; } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__14() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("class", 5, 5); -return x_1; +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; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__15() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__3; -x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__14; -x_3 = lean_string_append(x_1, x_2); -return x_3; } +else +{ +uint8_t x_40; +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_40 = !lean_is_exclusive(x_19); +if (x_40 == 0) +{ +return x_19; } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__16() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__15; -x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__6; -x_3 = lean_string_append(x_1, x_2); -return x_3; +lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_41 = lean_ctor_get(x_19, 0); +x_42 = lean_ctor_get(x_19, 1); +lean_inc(x_42); +lean_inc(x_41); +lean_dec(x_19); +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; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__17() { -_start: +} +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__16; -x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__14; -x_3 = lean_string_append(x_1, x_2); -return x_3; +uint8_t x_44; +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_44 = !lean_is_exclusive(x_13); +if (x_44 == 0) +{ +return x_13; +} +else +{ +lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_45 = lean_ctor_get(x_13, 0); +x_46 = lean_ctor_get(x_13, 1); +lean_inc(x_46); +lean_inc(x_45); +lean_dec(x_13); +x_47 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_47, 0, x_45); +lean_ctor_set(x_47, 1, x_46); +return x_47; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__18() { -_start: +} +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__17; -x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__9; -x_3 = lean_string_append(x_1, x_2); -return x_3; +uint8_t 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_2); +lean_dec(x_1); +x_48 = !lean_is_exclusive(x_10); +if (x_48 == 0) +{ +return x_10; +} +else +{ +lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_49 = lean_ctor_get(x_10, 0); +x_50 = lean_ctor_get(x_10, 1); +lean_inc(x_50); +lean_inc(x_49); +lean_dec(x_10); +x_51 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_51, 0, x_49); +lean_ctor_set(x_51, 1, x_50); +return x_51; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__19() { +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType(lean_object* x_1, lean_object* x_2, lean_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_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__18; -x_2 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; uint8_t x_14; lean_object* x_15; +x_9 = l_Lean_mkFreshId___at_Lean_Meta_mkFreshExprMVarAt___spec__2___rarg(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); +lean_inc(x_2); +x_12 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___boxed), 9, 3); +lean_closure_set(x_12, 0, x_3); +lean_closure_set(x_12, 1, x_1); +lean_closure_set(x_12, 2, x_2); +x_13 = 0; +x_14 = 0; +x_15 = l_Lean_Meta_withLocalDecl___at_Lean_Meta_GeneralizeTelescope_generalizeTelescopeAux___spec__1___rarg(x_10, x_13, x_2, x_12, x_14, x_4, x_5, x_6, x_7, x_11); +return x_15; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__20() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__1___boxed(lean_object* x_1, 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_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__19; -x_2 = l_Lean_MessageData_ofFormat(x_1); -return x_2; +lean_object* x_8; +x_8 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_8; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, 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_unsigned_to_nat(5u); -x_12 = l_Lean_Syntax_getArg(x_1, x_11); -x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Syntax_getArg(x_12, x_13); -lean_dec(x_12); -x_15 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__1; -x_16 = l_Lean_Syntax_isToken(x_15, x_14); -if (x_16 == 0) -{ -lean_object* x_17; lean_object* x_18; -lean_dec(x_14); -x_17 = lean_box(0); -x_18 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1(x_1, x_2, x_3, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_18; -} -else -{ -lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; lean_object* x_35; uint8_t x_36; lean_object* x_37; lean_object* x_38; -x_19 = l_Lean_Syntax_getArg(x_1, x_13); -lean_inc(x_19); -x_20 = l_Lean_Syntax_getKind(x_19); -x_21 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__3; -x_22 = lean_name_eq(x_20, x_21); -lean_dec(x_20); -x_23 = lean_ctor_get(x_8, 0); -x_24 = lean_ctor_get(x_8, 1); -x_25 = lean_ctor_get(x_8, 2); -x_26 = lean_ctor_get(x_8, 3); -x_27 = lean_ctor_get(x_8, 4); -x_28 = lean_ctor_get(x_8, 5); -x_29 = lean_ctor_get(x_8, 6); -x_30 = lean_ctor_get(x_8, 7); -x_31 = lean_ctor_get(x_8, 8); -x_32 = lean_ctor_get(x_8, 9); -x_33 = lean_ctor_get(x_8, 10); -x_34 = lean_ctor_get_uint8(x_8, sizeof(void*)*12); -x_35 = lean_ctor_get(x_8, 11); -x_36 = lean_ctor_get_uint8(x_8, sizeof(void*)*12 + 1); -x_37 = l_Lean_replaceRef(x_19, x_28); -lean_dec(x_19); -lean_inc(x_35); -lean_inc(x_33); -lean_inc(x_32); -lean_inc(x_31); -lean_inc(x_30); -lean_inc(x_29); -lean_inc(x_27); -lean_inc(x_26); -lean_inc(x_25); -lean_inc(x_24); -lean_inc(x_23); -x_38 = lean_alloc_ctor(0, 12, 2); -lean_ctor_set(x_38, 0, x_23); -lean_ctor_set(x_38, 1, x_24); -lean_ctor_set(x_38, 2, x_25); -lean_ctor_set(x_38, 3, x_26); -lean_ctor_set(x_38, 4, x_27); -lean_ctor_set(x_38, 5, x_37); -lean_ctor_set(x_38, 6, x_29); -lean_ctor_set(x_38, 7, x_30); -lean_ctor_set(x_38, 8, x_31); -lean_ctor_set(x_38, 9, x_32); -lean_ctor_set(x_38, 10, x_33); -lean_ctor_set(x_38, 11, x_35); -lean_ctor_set_uint8(x_38, sizeof(void*)*12, x_34); -lean_ctor_set_uint8(x_38, sizeof(void*)*12 + 1, x_36); -if (x_22 == 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; -x_39 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__13; -x_40 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__12; -x_41 = l_Lean_Linter_logLintIf___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__7(x_39, x_14, x_40, x_4, x_5, x_6, x_7, x_38, x_9, x_10); -lean_dec(x_14); -x_42 = lean_ctor_get(x_41, 0); -lean_inc(x_42); -x_43 = lean_ctor_get(x_41, 1); -lean_inc(x_43); -lean_dec(x_41); -x_44 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1(x_1, x_2, x_3, x_42, x_4, x_5, x_6, x_7, x_8, x_9, x_43); -lean_dec(x_42); -return x_44; -} -else -{ -lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_45 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__13; -x_46 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__20; -x_47 = l_Lean_Linter_logLintIf___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__7(x_45, x_14, x_46, x_4, x_5, x_6, x_7, x_38, x_9, x_10); -lean_dec(x_14); -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_Structure_0__Lean_Elab_Command_expandFields___lambda__1(x_1, x_2, x_3, x_48, x_4, x_5, x_6, x_7, x_8, x_9, x_49); -lean_dec(x_48); -return x_50; -} -} -} -} -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___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]; -_start: -{ -uint8_t x_19; lean_object* x_20; -x_19 = lean_unbox(x_5); -lean_dec(x_5); -x_20 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_19, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_11); -return x_20; -} -} -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___boxed(lean_object** _args) { -lean_object* x_1 = _args[0]; -lean_object* x_2 = _args[1]; -lean_object* x_3 = _args[2]; -lean_object* x_4 = _args[3]; -lean_object* x_5 = _args[4]; -lean_object* x_6 = _args[5]; -lean_object* x_7 = _args[6]; -lean_object* x_8 = _args[7]; -lean_object* x_9 = _args[8]; -lean_object* x_10 = _args[9]; -lean_object* x_11 = _args[10]; -lean_object* x_12 = _args[11]; -lean_object* x_13 = _args[12]; -lean_object* x_14 = _args[13]; -lean_object* x_15 = _args[14]; -lean_object* x_16 = _args[15]; -lean_object* x_17 = _args[16]; -_start: -{ -uint8_t x_18; size_t x_19; size_t x_20; lean_object* x_21; -x_18 = lean_unbox(x_2); -lean_dec(x_2); -x_19 = lean_unbox_usize(x_8); -lean_dec(x_8); -x_20 = lean_unbox_usize(x_9); -lean_dec(x_9); -x_21 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1(x_1, x_18, x_3, x_4, x_5, x_6, x_7, x_19, x_20, 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_7); -return x_21; -} -} -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; -x_9 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); -return x_9; -} -} -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; -x_10 = l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_8); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); +lean_dec(x_2); lean_dec(x_1); -return x_10; +return x_9; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___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_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___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_9; -x_9 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_7); -lean_dec(x_6); +lean_object* x_7; +x_7 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__3(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_9; +lean_dec(x_2); +lean_dec(x_1); +return x_7; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_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_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -uint8_t x_16; lean_object* x_17; -x_16 = lean_unbox(x_4); +lean_object* x_10; +x_10 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_4); -x_17 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__1(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); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); lean_dec(x_1); -return x_17; +return x_10; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -uint8_t x_14; lean_object* x_15; -x_14 = lean_unbox(x_4); -lean_dec(x_4); -x_15 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2(x_1, x_2, x_3, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_1); -return x_15; +lean_object* x_10; +x_10 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_3); +return x_10; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___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) { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_toVisibility___closed__1() { _start: { -uint8_t x_14; lean_object* x_15; -x_14 = lean_unbox(x_4); -lean_dec(x_4); -x_15 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3(x_1, x_2, x_3, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_6); -lean_dec(x_1); -return x_15; +lean_object* x_1; +x_1 = l_Lean_protectedExt; +return x_1; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_toVisibility(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -uint8_t x_15; lean_object* x_16; -x_15 = lean_unbox(x_4); -lean_dec(x_4); -x_16 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4(x_1, x_2, x_3, x_15, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_object* x_5; uint8_t x_6; +x_5 = lean_st_ref_get(x_3, x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_7 = lean_ctor_get(x_5, 0); +x_8 = lean_ctor_get(x_7, 0); +lean_inc(x_8); lean_dec(x_7); -lean_dec(x_6); +x_9 = lean_ctor_get(x_1, 1); +lean_inc(x_9); lean_dec(x_1); -return x_16; -} -} -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: +x_10 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_toVisibility___closed__1; +lean_inc(x_9); +x_11 = l_Lean_TagDeclarationExtension_isTagged(x_10, x_8, x_9); +lean_dec(x_8); +if (x_11 == 0) +{ +uint8_t x_12; +x_12 = l_Lean_isPrivateName(x_9); +lean_dec(x_9); +if (x_12 == 0) { uint8_t x_13; lean_object* x_14; -x_13 = lean_unbox(x_5); -lean_dec(x_5); -x_14 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5(x_1, x_2, x_3, x_4, x_13, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_4); -lean_dec(x_1); -return x_14; -} +x_13 = 0; +x_14 = lean_box(x_13); +lean_ctor_set(x_5, 0, x_14); +return x_5; } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, 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; -x_13 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___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); -lean_dec(x_5); -lean_dec(x_3); -return x_13; +uint8_t x_15; lean_object* x_16; +x_15 = 2; +x_16 = lean_box(x_15); +lean_ctor_set(x_5, 0, x_16); +return x_5; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { -_start: +else { -size_t x_14; size_t x_15; lean_object* x_16; -x_14 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_15 = lean_unbox_usize(x_5); -lean_dec(x_5); -x_16 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5(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); -lean_dec(x_1); -return x_16; +uint8_t x_17; lean_object* x_18; +lean_dec(x_9); +x_17 = 1; +x_18 = lean_box(x_17); +lean_ctor_set(x_5, 0, x_18); +return x_5; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___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: +else { -size_t x_14; size_t x_15; lean_object* x_16; -x_14 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_15 = lean_unbox_usize(x_5); +lean_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_5, 0); +x_20 = lean_ctor_get(x_5, 1); +lean_inc(x_20); +lean_inc(x_19); lean_dec(x_5); -x_16 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___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); +x_21 = lean_ctor_get(x_19, 0); +lean_inc(x_21); +lean_dec(x_19); +x_22 = lean_ctor_get(x_1, 1); +lean_inc(x_22); lean_dec(x_1); -return x_16; -} +x_23 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_toVisibility___closed__1; +lean_inc(x_22); +x_24 = l_Lean_TagDeclarationExtension_isTagged(x_23, x_21, x_22); +lean_dec(x_21); +if (x_24 == 0) +{ +uint8_t x_25; +x_25 = l_Lean_isPrivateName(x_22); +lean_dec(x_22); +if (x_25 == 0) +{ +uint8_t x_26; lean_object* x_27; lean_object* x_28; +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_20); +return x_28; } -LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___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: +else { -lean_object* x_11; -x_11 = l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___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); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); -return x_11; +uint8_t x_29; lean_object* x_30; lean_object* x_31; +x_29 = 2; +x_30 = lean_box(x_29); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_30); +lean_ctor_set(x_31, 1, x_20); +return x_31; } } -LEAN_EXPORT lean_object* l_Lean_Linter_logLintIf___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___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: +else { -lean_object* x_11; -x_11 = l_Lean_Linter_logLintIf___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__7(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_9); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); -return x_11; +uint8_t x_32; lean_object* x_33; lean_object* x_34; +lean_dec(x_22); +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_20); +return x_34; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -lean_object* x_12; -x_12 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___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_9); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -return x_12; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_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_Structure_0__Lean_Elab_Command_toVisibility___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___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_8); +lean_object* x_5; +x_5 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_toVisibility(x_1, x_2, x_3, x_4); +lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -return x_11; +return x_5; } } -LEAN_EXPORT uint8_t l___private_Lean_Elab_Structure_0__Lean_Elab_Command_validStructType(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reduceProjs___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) == 3) +lean_object* x_8; lean_object* x_9; +x_8 = lean_alloc_closure((void*)(l_Lean_NameSet_contains___boxed), 2, 1); +lean_closure_set(x_8, 0, x_1); +lean_inc(x_2); +x_9 = l_Lean_Meta_reduceProjOf_x3f(x_2, x_8, x_3, x_4, x_5, x_6, x_7); +if (lean_obj_tag(x_9) == 0) { -uint8_t x_2; -x_2 = 1; -return x_2; -} -else +lean_object* x_10; +x_10 = lean_ctor_get(x_9, 0); +lean_inc(x_10); +if (lean_obj_tag(x_10) == 0) { -uint8_t x_3; -x_3 = 0; -return x_3; -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_validStructType___boxed(lean_object* x_1) { -_start: +uint8_t x_11; +x_11 = !lean_is_exclusive(x_9); +if (x_11 == 0) { -uint8_t x_2; lean_object* x_3; -x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_validStructType(x_1); -lean_dec(x_1); -x_3 = lean_box(x_2); -return x_3; -} +lean_object* x_12; lean_object* x_13; +x_12 = lean_ctor_get(x_9, 0); +lean_dec(x_12); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_2); +lean_ctor_set(x_9, 0, x_13); +return x_9; } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6) { -_start: -{ -uint8_t x_7; -x_7 = lean_usize_dec_lt(x_5, x_4); -if (x_7 == 0) +else { -lean_inc(x_6); -return x_6; +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_9, 1); +lean_inc(x_14); +lean_dec(x_9); +x_15 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_15, 0, x_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); +return x_16; +} } else { -lean_object* x_8; lean_object* x_9; uint8_t x_10; -x_8 = lean_array_uget(x_3, x_5); -x_9 = lean_ctor_get(x_8, 0); -lean_inc(x_9); -x_10 = lean_name_eq(x_9, x_1); -lean_dec(x_9); -if (x_10 == 0) +uint8_t x_17; +lean_dec(x_2); +x_17 = !lean_is_exclusive(x_9); +if (x_17 == 0) { -size_t x_11; size_t x_12; -lean_dec(x_8); -x_11 = 1; -x_12 = lean_usize_add(x_5, x_11); +lean_object* x_18; uint8_t x_19; +x_18 = lean_ctor_get(x_9, 0); +lean_dec(x_18); +x_19 = !lean_is_exclusive(x_10); +if (x_19 == 0) { -size_t _tmp_4 = x_12; -lean_object* _tmp_5 = x_2; -x_5 = _tmp_4; -x_6 = _tmp_5; -} -goto _start; +lean_ctor_set_tag(x_10, 0); +return x_9; } else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_14 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_14, 0, x_8); -x_15 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_15, 0, x_14); -x_16 = lean_box(0); -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_15); -lean_ctor_set(x_17, 1, x_16); -return x_17; -} -} +lean_object* x_20; lean_object* x_21; +x_20 = lean_ctor_get(x_10, 0); +lean_inc(x_20); +lean_dec(x_10); +x_21 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_21, 0, x_20); +lean_ctor_set(x_9, 0, x_21); +return x_9; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___lambda__1(lean_object* x_1) { -_start: +else { -lean_object* x_2; -x_2 = lean_box(0); -return x_2; -} -} -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___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; -} +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_22 = lean_ctor_get(x_9, 1); +lean_inc(x_22); +lean_dec(x_9); +x_23 = lean_ctor_get(x_10, 0); +lean_inc(x_23); +if (lean_is_exclusive(x_10)) { + lean_ctor_release(x_10, 0); + x_24 = x_10; +} else { + lean_dec_ref(x_10); + x_24 = lean_box(0); } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___closed__2() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___lambda__1___boxed), 1, 0); -return x_1; +if (lean_is_scalar(x_24)) { + x_25 = lean_alloc_ctor(0, 1, 0); +} else { + x_25 = x_24; + lean_ctor_set_tag(x_25, 0); } +lean_ctor_set(x_25, 0, x_23); +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_22); +return x_26; } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___closed__2; -x_2 = lean_box(0); -x_3 = lean_apply_1(x_1, x_2); -return x_3; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f(lean_object* x_1, lean_object* x_2) { -_start: +else { -size_t x_3; size_t x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_3 = lean_array_size(x_1); -x_4 = 0; -x_5 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___closed__1; -x_6 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___spec__1(x_2, x_5, x_1, x_3, x_4, x_5); -x_7 = lean_ctor_get(x_6, 0); -lean_inc(x_7); -lean_dec(x_6); -if (lean_obj_tag(x_7) == 0) +uint8_t x_27; +lean_dec(x_2); +x_27 = !lean_is_exclusive(x_9); +if (x_27 == 0) { -lean_object* x_8; -x_8 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___closed__3; -return x_8; +return x_9; } else { -lean_object* x_9; -x_9 = lean_ctor_get(x_7, 0); -lean_inc(x_9); -lean_dec(x_7); -return x_9; +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_9, 0); +x_29 = lean_ctor_get(x_9, 1); +lean_inc(x_29); +lean_inc(x_28); +lean_dec(x_9); +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_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___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___private_Lean_Elab_Structure_0__Lean_Elab_Command_reduceProjs(lean_object* x_1, 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); -lean_dec(x_5); -x_9 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___spec__1(x_1, x_2, x_3, x_7, x_8, x_6); -lean_dec(x_6); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_9; +lean_object* x_8; lean_object* x_9; uint8_t x_10; lean_object* x_11; +x_8 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reduceProjs___lambda__1), 7, 1); +lean_closure_set(x_8, 0, x_2); +x_9 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___closed__1; +x_10 = 0; +x_11 = l_Lean_Meta_transform___at_Lean_Meta_zetaReduce___spec__1(x_1, x_9, x_8, x_10, x_10, x_3, x_4, x_5, x_6, x_7); +return x_11; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___lambda__1___boxed(lean_object* x_1) { +LEAN_EXPORT uint8_t l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___lambda__1(lean_object* x_1) { _start: { -lean_object* x_2; -x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___lambda__1(x_1); -lean_dec(x_1); +uint8_t x_2; +x_2 = 0; return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___boxed(lean_object* x_1, lean_object* x_2) { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___closed__1() { _start: { -lean_object* x_3; -x_3 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f(x_1, x_2); -lean_dec(x_2); -lean_dec(x_1); -return x_3; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___lambda__1___boxed), 1, 0); +return x_1; } } -LEAN_EXPORT uint8_t l___private_Lean_Elab_Structure_0__Lean_Elab_Command_containsFieldName(lean_object* x_1, lean_object* x_2) { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___closed__2() { _start: { -lean_object* x_3; -x_3 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f(x_1, x_2); -if (lean_obj_tag(x_3) == 0) -{ -uint8_t x_4; -x_4 = 0; -return x_4; -} -else -{ -uint8_t x_5; -lean_dec(x_3); -x_5 = 1; -return x_5; -} +lean_object* x_1; +x_1 = lean_mk_string_unchecked("ignoring default value for field '", 34, 34); +return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_containsFieldName___boxed(lean_object* x_1, lean_object* x_2) { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___closed__3() { _start: { -uint8_t x_3; lean_object* x_4; -x_3 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_containsFieldName(x_1, x_2); -lean_dec(x_2); -lean_dec(x_1); -x_4 = lean_box(x_3); -return x_4; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("' defined at '", 14, 14); +return x_1; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateFieldInfoVal___spec__1(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___closed__4() { _start: { -uint8_t x_6; -x_6 = lean_usize_dec_lt(x_4, x_3); -if (x_6 == 0) -{ -lean_dec(x_2); -return x_5; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("'", 1, 1); +return x_1; } -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; uint8_t x_13; uint8_t x_14; size_t x_15; size_t x_16; -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 = lean_ctor_get(x_7, 0); -lean_inc(x_10); -x_11 = lean_ctor_get(x_7, 1); -lean_inc(x_11); -x_12 = lean_ctor_get(x_7, 2); -lean_inc(x_12); -x_13 = lean_ctor_get_uint8(x_7, sizeof(void*)*4); -x_14 = lean_name_eq(x_10, x_1); -x_15 = 1; -x_16 = lean_usize_add(x_4, x_15); -if (x_14 == 0) -{ -lean_object* x_17; -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -x_17 = lean_array_uset(x_9, x_4, x_7); -x_4 = x_16; -x_5 = x_17; -goto _start; } -else +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed(lean_object* x_1, lean_object* x_2, lean_object* x_3, 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_19; -x_19 = !lean_is_exclusive(x_7); -if (x_19 == 0) +uint8_t x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; +x_10 = 1; +x_11 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___closed__1; +x_12 = l_Lean_Name_toString(x_2, x_10, x_11); +x_13 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___closed__2; +x_14 = lean_string_append(x_13, x_12); +lean_dec(x_12); +x_15 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___closed__3; +x_16 = lean_string_append(x_14, x_15); +x_17 = l_Lean_Name_toString(x_1, x_10, x_11); +x_18 = lean_string_append(x_16, x_17); +lean_dec(x_17); +x_19 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___closed__4; +x_20 = lean_string_append(x_18, x_19); +x_21 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_21, 0, x_20); +x_22 = l_Lean_MessageData_ofFormat(x_21); +x_23 = l_Lean_logWarning___at_Lean_Elab_Term_mkConst___spec__4(x_22, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_24 = !lean_is_exclusive(x_23); +if (x_24 == 0) { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_20 = lean_ctor_get(x_7, 3); -lean_dec(x_20); -x_21 = lean_ctor_get(x_7, 2); -lean_dec(x_21); -x_22 = lean_ctor_get(x_7, 1); -lean_dec(x_22); -x_23 = lean_ctor_get(x_7, 0); -lean_dec(x_23); -lean_inc(x_2); -x_24 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_24, 0, x_2); -lean_ctor_set(x_7, 3, x_24); -x_25 = lean_array_uset(x_9, x_4, x_7); -x_4 = x_16; -x_5 = x_25; -goto _start; +lean_object* x_25; lean_object* x_26; +x_25 = lean_ctor_get(x_23, 0); +lean_dec(x_25); +x_26 = lean_box(0); +lean_ctor_set(x_23, 0, x_26); +return x_23; } else { lean_object* x_27; lean_object* x_28; lean_object* x_29; -lean_dec(x_7); -lean_inc(x_2); -x_27 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_27, 0, x_2); -x_28 = lean_alloc_ctor(0, 4, 1); -lean_ctor_set(x_28, 0, x_10); -lean_ctor_set(x_28, 1, x_11); -lean_ctor_set(x_28, 2, x_12); -lean_ctor_set(x_28, 3, x_27); -lean_ctor_set_uint8(x_28, sizeof(void*)*4, x_13); -x_29 = lean_array_uset(x_9, x_4, x_28); -x_4 = x_16; -x_5 = x_29; -goto _start; +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_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___lambda__1___boxed(lean_object* x_1) { +_start: +{ +uint8_t x_2; lean_object* x_3; +x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___lambda__1(x_1); +lean_dec(x_1); +x_3 = lean_box(x_2); +return x_3; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateFieldInfoVal(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, 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_4; size_t x_5; lean_object* x_6; -x_4 = lean_array_size(x_1); -x_5 = 0; -x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateFieldInfoVal___spec__1(x_2, x_3, x_4, x_5, x_1); -return x_6; +lean_object* x_10; +x_10 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed(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_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateFieldInfoVal___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_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateFieldInfoVal___spec__1(x_1, x_2, x_6, x_7, x_5); -lean_dec(x_1); -return x_8; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateFieldInfoVal___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateFieldInfoVal(x_1, x_2, x_3); -lean_dec(x_2); -return x_4; -} -} -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__1() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_go_x3f___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("structureDiamondWarning", 23, 23); +x_1 = lean_mk_string_unchecked("id", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__2() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_go_x3f___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__1; +x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_go_x3f___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__3() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_go_x3f(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("enable/disable warning messages for structure diamonds", 54, 54); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__4() { -_start: +if (lean_obj_tag(x_5) == 6) { -uint8_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = 0; -x_2 = l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__3; -x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__3; -x_4 = lean_box(x_1); -x_5 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_5, 0, x_4); -lean_ctor_set(x_5, 1, x_2); -lean_ctor_set(x_5, 2, x_3); -return x_5; -} -} -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__5() { -_start: +lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; uint8_t x_17; +x_13 = lean_ctor_get(x_5, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_5, 1); +lean_inc(x_14); +x_15 = lean_ctor_get(x_5, 2); +lean_inc(x_15); +x_16 = lean_ctor_get_uint8(x_5, sizeof(void*)*3 + 8); +lean_dec(x_5); +x_17 = l_Lean_BinderInfo_isExplicit(x_16); +if (x_17 == 0) { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Elab", 4, 4); -return x_1; -} +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_dec(x_13); +x_18 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_18, 0, x_14); +x_19 = 0; +x_20 = lean_box(0); +lean_inc(x_8); +x_21 = l___private_Lean_Meta_Basic_0__Lean_Meta_mkFreshExprMVarImpl(x_18, x_19, x_20, x_8, x_9, x_10, x_11, 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 = lean_expr_instantiate1(x_15, x_22); +lean_dec(x_22); +lean_dec(x_15); +x_5 = x_24; +x_12 = x_23; +goto _start; } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____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_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__1; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__5; -x_3 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__1; -x_4 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__1; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990_(lean_object* x_1) { -_start: +lean_object* x_26; +x_26 = l_Lean_RBNode_find___at_Lean_NameMap_find_x3f___spec__1___rarg(x_1, x_13); +lean_dec(x_13); +if (lean_obj_tag(x_26) == 0) { -lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__2; -x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__4; -x_4 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__6; -x_5 = l_Lean_Option_register___at_Lean_Elab_initFn____x40_Lean_Elab_AutoBound___hyg_6____spec__1(x_2, x_3, x_4, x_1); -return x_5; -} +lean_object* x_27; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_2); +x_27 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed(x_3, x_4, 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); +return x_27; } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +else { -uint8_t x_10; -x_10 = lean_usize_dec_lt(x_5, x_4); -if (x_10 == 0) +lean_object* x_28; lean_object* x_29; +x_28 = lean_ctor_get(x_26, 0); +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_28); +x_29 = lean_infer_type(x_28, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_29) == 0) { -lean_object* x_11; +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_29, 0); +lean_inc(x_30); +x_31 = lean_ctor_get(x_29, 1); +lean_inc(x_31); +lean_dec(x_29); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +x_32 = l_Lean_Meta_isExprDefEq(x_30, x_14, x_8, x_9, x_10, x_11, x_31); +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) +{ +lean_object* x_35; lean_object* x_36; +lean_dec(x_28); +lean_dec(x_15); lean_dec(x_2); -x_11 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_11, 0, x_6); -lean_ctor_set(x_11, 1, x_9); -return x_11; +x_35 = lean_ctor_get(x_32, 1); +lean_inc(x_35); +lean_dec(x_32); +x_36 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed(x_3, x_4, x_6, x_7, x_8, x_9, x_10, x_11, x_35); +lean_dec(x_11); +lean_dec(x_9); +lean_dec(x_8); +return x_36; } else { -lean_object* x_12; uint8_t x_13; -lean_dec(x_6); -x_12 = lean_array_uget(x_3, x_5); -x_13 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_containsFieldName(x_1, x_12); -if (x_13 == 0) +lean_object* x_37; lean_object* x_38; +x_37 = lean_ctor_get(x_32, 1); +lean_inc(x_37); +lean_dec(x_32); +x_38 = lean_expr_instantiate1(x_15, x_28); +lean_dec(x_28); +lean_dec(x_15); +x_5 = x_38; +x_12 = x_37; +goto _start; +} +} +else { -size_t x_14; size_t x_15; -lean_dec(x_12); -x_14 = 1; -x_15 = lean_usize_add(x_5, x_14); -lean_inc(x_2); +uint8_t x_40; +lean_dec(x_28); +lean_dec(x_15); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_40 = !lean_is_exclusive(x_32); +if (x_40 == 0) { -size_t _tmp_4 = x_15; -lean_object* _tmp_5 = x_2; -x_5 = _tmp_4; -x_6 = _tmp_5; +return x_32; +} +else +{ +lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_41 = lean_ctor_get(x_32, 0); +x_42 = lean_ctor_get(x_32, 1); +lean_inc(x_42); +lean_inc(x_41); +lean_dec(x_32); +x_43 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_43, 0, x_41); +lean_ctor_set(x_43, 1, x_42); +return x_43; +} } -goto _start; } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +uint8_t x_44; +lean_dec(x_28); +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_4); +lean_dec(x_3); lean_dec(x_2); -x_17 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_17, 0, x_12); -x_18 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_18, 0, x_17); -x_19 = lean_box(0); -x_20 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_20, 0, x_18); -lean_ctor_set(x_20, 1, x_19); -x_21 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_21, 0, x_20); -lean_ctor_set(x_21, 1, x_9); -return x_21; +x_44 = !lean_is_exclusive(x_29); +if (x_44 == 0) +{ +return x_29; } +else +{ +lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_45 = lean_ctor_get(x_29, 0); +x_46 = lean_ctor_get(x_29, 1); +lean_inc(x_46); +lean_inc(x_45); +lean_dec(x_29); +x_47 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_47, 0, x_45); +lean_ctor_set(x_47, 1, x_46); +return x_47; } } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f___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; -x_6 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_6, 0, x_1); -lean_ctor_set(x_6, 1, x_5); -return x_6; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f(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; uint8_t x_10; lean_object* x_11; lean_object* x_12; size_t x_13; size_t x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_6 = lean_st_ref_get(x_4, x_5); -x_7 = lean_ctor_get(x_6, 0); -lean_inc(x_7); -x_8 = lean_ctor_get(x_6, 1); -lean_inc(x_8); -lean_dec(x_6); -x_9 = lean_ctor_get(x_7, 0); -lean_inc(x_9); -lean_dec(x_7); -x_10 = 1; -x_11 = l_Lean_getStructureFieldsFlattened(x_9, x_2, x_10); -lean_dec(x_9); -x_12 = lean_box(0); -x_13 = lean_array_size(x_11); -x_14 = 0; -x_15 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___closed__1; -x_16 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f___spec__1(x_1, x_15, x_11, x_13, x_14, x_15, x_3, x_4, x_8); -lean_dec(x_11); -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -lean_dec(x_17); -if (lean_obj_tag(x_18) == 0) +lean_object* x_48; lean_object* x_49; uint8_t x_50; +lean_dec(x_4); +lean_dec(x_3); +x_48 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_go_x3f___closed__2; +x_49 = lean_unsigned_to_nat(2u); +x_50 = l_Lean_Expr_isAppOfArity(x_5, x_48, x_49); +if (x_50 == 0) { -uint8_t x_19; -x_19 = !lean_is_exclusive(x_16); -if (x_19 == 0) +lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_51 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +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___private_Lean_Elab_Structure_0__Lean_Elab_Command_reduceProjs(x_52, x_2, x_8, x_9, x_10, x_11, x_53); +if (lean_obj_tag(x_54) == 0) { -lean_object* x_20; -x_20 = lean_ctor_get(x_16, 0); -lean_dec(x_20); -lean_ctor_set(x_16, 0, x_12); -return x_16; +uint8_t x_55; +x_55 = !lean_is_exclusive(x_54); +if (x_55 == 0) +{ +lean_object* x_56; lean_object* x_57; +x_56 = lean_ctor_get(x_54, 0); +x_57 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_57, 0, x_56); +lean_ctor_set(x_54, 0, x_57); +return x_54; } else { -lean_object* x_21; lean_object* x_22; -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_12); -lean_ctor_set(x_22, 1, x_21); -return x_22; +lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; +x_58 = lean_ctor_get(x_54, 0); +x_59 = lean_ctor_get(x_54, 1); +lean_inc(x_59); +lean_inc(x_58); +lean_dec(x_54); +x_60 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_60, 0, x_58); +x_61 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_61, 0, x_60); +lean_ctor_set(x_61, 1, x_59); +return x_61; } } else { -uint8_t x_23; -x_23 = !lean_is_exclusive(x_16); -if (x_23 == 0) +uint8_t x_62; +x_62 = !lean_is_exclusive(x_54); +if (x_62 == 0) { -lean_object* x_24; lean_object* x_25; -x_24 = lean_ctor_get(x_16, 0); -lean_dec(x_24); -x_25 = lean_ctor_get(x_18, 0); -lean_inc(x_25); -lean_dec(x_18); -lean_ctor_set(x_16, 0, x_25); -return x_16; +return x_54; } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_16, 1); -lean_inc(x_26); -lean_dec(x_16); -x_27 = lean_ctor_get(x_18, 0); -lean_inc(x_27); -lean_dec(x_18); -x_28 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_28, 0, x_27); -lean_ctor_set(x_28, 1, x_26); -return x_28; -} +lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_63 = lean_ctor_get(x_54, 0); +x_64 = lean_ctor_get(x_54, 1); +lean_inc(x_64); +lean_inc(x_63); +lean_dec(x_54); +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_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +else { -size_t x_10; size_t x_11; lean_object* x_12; -x_10 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_11 = lean_unbox_usize(x_5); +lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; +x_66 = l_Lean_Expr_appArg_x21(x_5); lean_dec(x_5); -x_12 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f___spec__1(x_1, x_2, x_3, x_10, x_11, x_6, x_7, x_8, x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_1); -return x_12; -} +x_67 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_66, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +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 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reduceProjs(x_68, x_2, x_8, x_9, x_10, x_11, x_69); +if (lean_obj_tag(x_70) == 0) +{ +uint8_t x_71; +x_71 = !lean_is_exclusive(x_70); +if (x_71 == 0) +{ +lean_object* x_72; lean_object* x_73; +x_72 = lean_ctor_get(x_70, 0); +x_73 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_73, 0, x_72); +lean_ctor_set(x_70, 0, x_73); +return x_70; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f___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___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f___lambda__1(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_6; +lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; +x_74 = lean_ctor_get(x_70, 0); +x_75 = lean_ctor_get(x_70, 1); +lean_inc(x_75); +lean_inc(x_74); +lean_dec(x_70); +x_76 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_76, 0, x_74); +x_77 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_77, 0, x_76); +lean_ctor_set(x_77, 1, x_75); +return x_77; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f___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___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -return x_6; +uint8_t x_78; +x_78 = !lean_is_exclusive(x_70); +if (x_78 == 0) +{ +return x_70; +} +else +{ +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; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_go_x3f___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; -lean_inc(x_2); -lean_inc(x_1); -x_17 = l_Lean_Name_append(x_1, x_2); -x_18 = lean_box(0); -x_19 = 2; -x_20 = lean_alloc_ctor(0, 4, 1); -lean_ctor_set(x_20, 0, x_2); -lean_ctor_set(x_20, 1, x_17); -lean_ctor_set(x_20, 2, x_9); -lean_ctor_set(x_20, 3, x_18); -lean_ctor_set_uint8(x_20, sizeof(void*)*4, x_19); -x_21 = lean_array_push(x_3, x_20); -x_22 = lean_unsigned_to_nat(1u); -x_23 = lean_nat_add(x_4, x_22); -x_24 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg(x_1, x_5, x_6, x_7, x_8, x_23, x_21, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -return x_24; +lean_object* x_13; +x_13 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_go_x3f(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_1); +return x_13; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_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, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_17; -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_2); -lean_inc(x_1); -x_17 = l_Lean_Meta_mkProjection(x_1, x_2, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_17) == 0) +lean_object* x_12; uint8_t x_13; +x_12 = lean_st_ref_get(x_10, x_11); +x_13 = !lean_is_exclusive(x_12); +if (x_13 == 0) { -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_17, 1); -lean_inc(x_19); -lean_dec(x_17); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_18); -x_20 = lean_infer_type(x_18, x_12, x_13, x_14, x_15, x_19); -if (lean_obj_tag(x_20) == 0) +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_14 = lean_ctor_get(x_12, 0); +x_15 = lean_ctor_get(x_12, 1); +x_16 = lean_ctor_get(x_14, 0); +lean_inc(x_16); +lean_dec(x_14); +lean_inc(x_4); +lean_inc(x_3); +x_17 = l_Lean_getDefaultFnForField_x3f(x_16, x_3, x_4); +if (lean_obj_tag(x_17) == 0) { -lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; lean_object* x_25; -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_20, 1); -lean_inc(x_22); -lean_dec(x_20); -lean_inc(x_2); -x_23 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___lambda__1___boxed), 16, 8); -lean_closure_set(x_23, 0, x_3); -lean_closure_set(x_23, 1, x_2); -lean_closure_set(x_23, 2, x_4); -lean_closure_set(x_23, 3, x_5); -lean_closure_set(x_23, 4, x_1); -lean_closure_set(x_23, 5, x_6); -lean_closure_set(x_23, 6, x_7); -lean_closure_set(x_23, 7, x_8); -x_24 = 0; -x_25 = l_Lean_Meta_withLetDecl___at_Lean_Elab_Term_elabLetDeclAux___spec__2___rarg(x_2, x_21, x_18, x_23, x_24, x_10, x_11, x_12, x_13, x_14, x_15, x_22); -return x_25; -} -else -{ -uint8_t x_26; -lean_dec(x_18); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); +lean_object* 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); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_26 = !lean_is_exclusive(x_20); -if (x_26 == 0) -{ -return x_20; +x_18 = lean_box(0); +lean_ctor_set(x_12, 0, x_18); +return x_12; } else { +lean_object* x_19; lean_object* x_20; +lean_free_object(x_12); +x_19 = lean_ctor_get(x_17, 0); +lean_inc(x_19); +lean_dec(x_17); +lean_inc(x_5); +x_20 = l_Lean_getConstInfo___at_Lean_Elab_Term_mkConst___spec__1(x_19, x_5, x_6, x_7, x_8, x_9, x_10, x_15); +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; +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_Meta_mkFreshLevelMVarsFor(x_21, x_7, x_8, x_9, x_10, x_22); +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +x_26 = l_Lean_Core_instantiateValueLevelParams(x_21, x_24, x_9, x_10, x_25); +lean_dec(x_21); +if (lean_obj_tag(x_26) == 0) +{ lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_20, 0); -x_28 = lean_ctor_get(x_20, 1); -lean_inc(x_28); +x_27 = lean_ctor_get(x_26, 0); lean_inc(x_27); -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); +x_28 = lean_ctor_get(x_26, 1); +lean_inc(x_28); +lean_dec(x_26); +x_29 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_go_x3f(x_1, x_2, x_3, x_4, x_27, x_5, x_6, x_7, x_8, x_9, x_10, x_28); +lean_dec(x_5); return x_29; } -} -} else { uint8_t x_30; -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); lean_dec(x_10); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_30 = !lean_is_exclusive(x_17); +x_30 = !lean_is_exclusive(x_26); if (x_30 == 0) { -return x_17; +return x_26; } else { lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_31 = lean_ctor_get(x_17, 0); -x_32 = lean_ctor_get(x_17, 1); +x_31 = lean_ctor_get(x_26, 0); +x_32 = lean_ctor_get(x_26, 1); lean_inc(x_32); lean_inc(x_31); -lean_dec(x_17); +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); @@ -11204,6481 +10800,4198 @@ return x_33; } } } -} -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("field '", 7, 7); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__3() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("' from '", 8, 8); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__4() { -_start: +uint8_t x_34; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_34 = !lean_is_exclusive(x_20); +if (x_34 == 0) { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__3; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} +return x_20; } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__5() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("' has already been declared", 27, 27); -return x_1; +lean_object* x_35; lean_object* x_36; lean_object* x_37; +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_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +return x_37; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__5; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { -_start: +else { -lean_object* x_15; uint8_t x_16; -x_15 = lean_array_get_size(x_4); -x_16 = lean_nat_dec_lt(x_6, x_15); -lean_dec(x_15); -if (x_16 == 0) +lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_38 = lean_ctor_get(x_12, 0); +x_39 = lean_ctor_get(x_12, 1); +lean_inc(x_39); +lean_inc(x_38); +lean_dec(x_12); +x_40 = lean_ctor_get(x_38, 0); +lean_inc(x_40); +lean_dec(x_38); +lean_inc(x_4); +lean_inc(x_3); +x_41 = l_Lean_getDefaultFnForField_x3f(x_40, x_3, x_4); +if (lean_obj_tag(x_41) == 0) { -lean_object* x_17; -lean_dec(x_6); +lean_object* x_42; lean_object* x_43; +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_17 = lean_apply_8(x_5, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -return x_17; +x_42 = lean_box(0); +x_43 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_43, 0, x_42); +lean_ctor_set(x_43, 1, x_39); +return x_43; } else { -lean_object* x_18; uint8_t x_19; -x_18 = lean_array_fget(x_4, x_6); -x_19 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_containsFieldName(x_7, x_18); -if (x_19 == 0) +lean_object* x_44; lean_object* x_45; +x_44 = lean_ctor_get(x_41, 0); +lean_inc(x_44); +lean_dec(x_41); +lean_inc(x_5); +x_45 = l_Lean_getConstInfo___at_Lean_Elab_Term_mkConst___spec__1(x_44, x_5, x_6, x_7, x_8, x_9, x_10, x_39); +if (lean_obj_tag(x_45) == 0) { -lean_object* x_20; lean_object* x_21; -x_20 = lean_box(0); -x_21 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___lambda__2(x_2, x_18, x_1, x_7, x_6, x_3, x_4, x_5, x_20, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -return x_21; +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_46 = lean_ctor_get(x_45, 0); +lean_inc(x_46); +x_47 = lean_ctor_get(x_45, 1); +lean_inc(x_47); +lean_dec(x_45); +x_48 = l_Lean_Meta_mkFreshLevelMVarsFor(x_46, x_7, x_8, x_9, x_10, 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 = l_Lean_Core_instantiateValueLevelParams(x_46, x_49, x_9, x_10, x_50); +lean_dec(x_46); +if (lean_obj_tag(x_51) == 0) +{ +lean_object* x_52; lean_object* x_53; lean_object* 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___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_go_x3f(x_1, x_2, x_3, x_4, x_52, x_5, x_6, x_7, x_8, x_9, x_10, x_53); +lean_dec(x_5); +return x_54; } 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; uint8_t x_32; +lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_22 = l_Lean_MessageData_ofName(x_18); -x_23 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__2; -x_24 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_24, 0, x_23); -lean_ctor_set(x_24, 1, x_22); -x_25 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__4; -x_26 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_26, 0, x_24); -lean_ctor_set(x_26, 1, x_25); -x_27 = l_Lean_MessageData_ofName(x_3); -x_28 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_28, 0, x_26); -lean_ctor_set(x_28, 1, x_27); -x_29 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__6; -x_30 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_30, 0, x_28); -lean_ctor_set(x_30, 1, x_29); -x_31 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_30, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -x_32 = !lean_is_exclusive(x_31); -if (x_32 == 0) -{ -return x_31; -} -else -{ -lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_33 = lean_ctor_get(x_31, 0); -x_34 = lean_ctor_get(x_31, 1); -lean_inc(x_34); -lean_inc(x_33); -lean_dec(x_31); -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_55 = lean_ctor_get(x_51, 0); +lean_inc(x_55); +x_56 = lean_ctor_get(x_51, 1); +lean_inc(x_56); +if (lean_is_exclusive(x_51)) { + lean_ctor_release(x_51, 0); + lean_ctor_release(x_51, 1); + x_57 = x_51; +} else { + lean_dec_ref(x_51); + 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_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg), 14, 0); -return x_2; +lean_ctor_set(x_58, 0, x_55); +lean_ctor_set(x_58, 1, x_56); +return x_58; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: +else { -lean_object* x_17; -x_17 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +lean_object* x_59; lean_object* x_60; 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_5); lean_dec(x_4); -return x_17; -} +lean_dec(x_3); +lean_dec(x_2); +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; +} else { + lean_dec_ref(x_45); + x_61 = lean_box(0); } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_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, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: -{ -lean_object* x_17; -x_17 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_9); -return x_17; +if (lean_is_scalar(x_61)) { + x_62 = lean_alloc_ctor(1, 2, 0); +} else { + x_62 = x_61; } +lean_ctor_set(x_62, 0, x_59); +lean_ctor_set(x_62, 1, x_60); +return x_62; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields___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) { -_start: -{ -lean_object* x_14; lean_object* x_15; -x_14 = lean_unsigned_to_nat(0u); -x_15 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg(x_1, x_2, x_3, x_4, x_6, x_14, x_5, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -return x_15; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields___rarg), 13, 0); -return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getNestedProjectionArg___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___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_8; -x_8 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_8, 0, x_1); -lean_ctor_set(x_8, 1, x_7); -return x_8; +lean_object* x_12; +x_12 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_6); +lean_dec(x_1); +return x_12; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getNestedProjectionArg(lean_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___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_processOveriddenDefaultValues___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -lean_object* x_7; -x_7 = l_Lean_Expr_getAppFn(x_1); -if (lean_obj_tag(x_7) == 4) -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; -x_8 = lean_ctor_get(x_7, 0); -lean_inc(x_8); -lean_dec(x_7); -x_9 = l_Lean_getProjectionFnInfo_x3f___at_Lean_Meta_getStuckMVar_x3f___spec__1(x_8, x_2, x_3, x_4, x_5, x_6); -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) +uint8_t x_14; +x_14 = lean_usize_dec_lt(x_5, x_4); +if (x_14 == 0) { -lean_object* x_12; -x_12 = lean_ctor_get(x_9, 0); +lean_object* x_15; lean_dec(x_12); -lean_ctor_set(x_9, 0, x_1); -return x_9; -} -else -{ -lean_object* x_13; lean_object* x_14; -x_13 = lean_ctor_get(x_9, 1); -lean_inc(x_13); +lean_dec(x_11); +lean_dec(x_10); lean_dec(x_9); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_1); -lean_ctor_set(x_14, 1, x_13); -return x_14; -} +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +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_15; uint8_t x_16; -x_15 = lean_ctor_get(x_10, 0); -lean_inc(x_15); -lean_dec(x_10); -x_16 = !lean_is_exclusive(x_9); -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; uint8_t x_24; -x_17 = lean_ctor_get(x_9, 1); -x_18 = lean_ctor_get(x_9, 0); -lean_dec(x_18); -x_19 = lean_ctor_get(x_15, 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_object* x_22; uint8_t x_23; lean_object* x_24; +x_16 = lean_array_uget(x_6, x_5); +x_17 = lean_unsigned_to_nat(0u); +x_18 = lean_array_uset(x_6, x_5, x_17); +x_19 = lean_ctor_get(x_16, 0); lean_inc(x_19); -lean_dec(x_15); -x_20 = lean_unsigned_to_nat(0u); -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); -x_24 = lean_nat_dec_eq(x_21, x_23); -lean_dec(x_23); -lean_dec(x_21); -if (x_24 == 0) +x_20 = lean_ctor_get(x_16, 1); +lean_inc(x_20); +x_21 = lean_ctor_get(x_16, 2); +lean_inc(x_21); +x_22 = lean_ctor_get(x_16, 3); +lean_inc(x_22); +x_23 = lean_ctor_get_uint8(x_16, sizeof(void*)*5); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_7); +lean_inc(x_20); +lean_inc(x_3); +lean_inc(x_2); +x_24 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f(x_1, x_2, x_3, x_20, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_24) == 0) { -lean_ctor_set(x_9, 0, x_1); -return x_9; +lean_object* x_25; +x_25 = lean_ctor_get(x_24, 0); +lean_inc(x_25); +if (lean_obj_tag(x_25) == 0) +{ +lean_object* x_26; size_t x_27; size_t x_28; lean_object* x_29; +lean_dec(x_22); +lean_dec(x_21); +lean_dec(x_20); +lean_dec(x_19); +x_26 = lean_ctor_get(x_24, 1); +lean_inc(x_26); +lean_dec(x_24); +x_27 = 1; +x_28 = lean_usize_add(x_5, x_27); +x_29 = lean_array_uset(x_18, x_5, x_16); +x_5 = x_28; +x_6 = x_29; +x_13 = x_26; +goto _start; } else { -lean_object* x_25; lean_object* x_26; uint8_t x_27; -lean_free_object(x_9); -x_25 = l_Lean_Expr_appArg_x21(x_1); -lean_dec(x_1); -x_26 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getNestedProjectionArg(x_25, x_2, x_3, x_4, x_5, x_17); -x_27 = !lean_is_exclusive(x_26); -if (x_27 == 0) +uint8_t x_31; +x_31 = !lean_is_exclusive(x_16); +if (x_31 == 0) { -return x_26; +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; uint8_t x_38; +x_32 = lean_ctor_get(x_16, 4); +lean_dec(x_32); +x_33 = lean_ctor_get(x_16, 3); +lean_dec(x_33); +x_34 = lean_ctor_get(x_16, 2); +lean_dec(x_34); +x_35 = lean_ctor_get(x_16, 1); +lean_dec(x_35); +x_36 = lean_ctor_get(x_16, 0); +lean_dec(x_36); +x_37 = lean_ctor_get(x_24, 1); +lean_inc(x_37); +lean_dec(x_24); +x_38 = !lean_is_exclusive(x_25); +if (x_38 == 0) +{ +size_t x_39; size_t x_40; lean_object* x_41; +lean_ctor_set(x_16, 4, x_25); +x_39 = 1; +x_40 = lean_usize_add(x_5, x_39); +x_41 = lean_array_uset(x_18, x_5, x_16); +x_5 = x_40; +x_6 = x_41; +x_13 = x_37; +goto _start; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_28 = lean_ctor_get(x_26, 0); -x_29 = lean_ctor_get(x_26, 1); -lean_inc(x_29); -lean_inc(x_28); -lean_dec(x_26); -x_30 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_30, 0, x_28); -lean_ctor_set(x_30, 1, x_29); -return x_30; +lean_object* x_43; lean_object* x_44; size_t x_45; size_t x_46; lean_object* x_47; +x_43 = lean_ctor_get(x_25, 0); +lean_inc(x_43); +lean_dec(x_25); +x_44 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_44, 0, x_43); +lean_ctor_set(x_16, 4, x_44); +x_45 = 1; +x_46 = lean_usize_add(x_5, x_45); +x_47 = lean_array_uset(x_18, x_5, x_16); +x_5 = x_46; +x_6 = x_47; +x_13 = x_37; +goto _start; +} +} +else +{ +lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; size_t x_54; size_t x_55; lean_object* x_56; +lean_dec(x_16); +x_49 = lean_ctor_get(x_24, 1); +lean_inc(x_49); +lean_dec(x_24); +x_50 = lean_ctor_get(x_25, 0); +lean_inc(x_50); +if (lean_is_exclusive(x_25)) { + lean_ctor_release(x_25, 0); + x_51 = x_25; +} else { + lean_dec_ref(x_25); + x_51 = lean_box(0); +} +if (lean_is_scalar(x_51)) { + x_52 = lean_alloc_ctor(1, 1, 0); +} else { + x_52 = x_51; +} +lean_ctor_set(x_52, 0, x_50); +x_53 = lean_alloc_ctor(0, 5, 1); +lean_ctor_set(x_53, 0, x_19); +lean_ctor_set(x_53, 1, x_20); +lean_ctor_set(x_53, 2, x_21); +lean_ctor_set(x_53, 3, x_22); +lean_ctor_set(x_53, 4, x_52); +lean_ctor_set_uint8(x_53, sizeof(void*)*5, x_23); +x_54 = 1; +x_55 = lean_usize_add(x_5, x_54); +x_56 = lean_array_uset(x_18, x_5, x_53); +x_5 = x_55; +x_6 = x_56; +x_13 = x_49; +goto _start; } } } else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; -x_31 = lean_ctor_get(x_9, 1); -lean_inc(x_31); +uint8_t x_58; +lean_dec(x_22); +lean_dec(x_21); +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_16); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); lean_dec(x_9); -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___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); -x_37 = lean_nat_dec_eq(x_34, x_36); -lean_dec(x_36); -lean_dec(x_34); -if (x_37 == 0) +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +x_58 = !lean_is_exclusive(x_24); +if (x_58 == 0) { -lean_object* x_38; -x_38 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_38, 0, x_1); -lean_ctor_set(x_38, 1, x_31); -return x_38; +return x_24; } 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; -x_39 = l_Lean_Expr_appArg_x21(x_1); -lean_dec(x_1); -x_40 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getNestedProjectionArg(x_39, x_2, x_3, x_4, x_5, x_31); -x_41 = lean_ctor_get(x_40, 0); -lean_inc(x_41); -x_42 = lean_ctor_get(x_40, 1); -lean_inc(x_42); -if (lean_is_exclusive(x_40)) { - lean_ctor_release(x_40, 0); - lean_ctor_release(x_40, 1); - x_43 = x_40; -} else { - lean_dec_ref(x_40); - x_43 = lean_box(0); -} -if (lean_is_scalar(x_43)) { - x_44 = lean_alloc_ctor(0, 2, 0); -} else { - x_44 = x_43; +lean_object* x_59; lean_object* x_60; lean_object* x_61; +x_59 = lean_ctor_get(x_24, 0); +x_60 = lean_ctor_get(x_24, 1); +lean_inc(x_60); +lean_inc(x_59); +lean_dec(x_24); +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_ctor_set(x_44, 0, x_41); -lean_ctor_set(x_44, 1, x_42); -return x_44; } } } } -else +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_processOveriddenDefaultValues(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, 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_45; -lean_dec(x_7); -x_45 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_45, 0, x_1); -lean_ctor_set(x_45, 1, x_6); -return x_45; +size_t x_12; size_t x_13; lean_object* x_14; +x_12 = lean_array_size(x_1); +x_13 = 0; +x_14 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_processOveriddenDefaultValues___spec__1(x_2, x_3, x_4, x_12, x_13, x_1, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_14; } } +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_processOveriddenDefaultValues___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +size_t x_14; size_t x_15; lean_object* x_16; +x_14 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_15 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_16 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_processOveriddenDefaultValues___spec__1(x_1, x_2, x_3, x_14, x_15, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_8); +lean_dec(x_1); +return x_16; +} } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getNestedProjectionArg___lambda__1___boxed(lean_object* x_1, lean_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_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_processOveriddenDefaultValues___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, 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; -x_8 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getNestedProjectionArg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_object* x_12; +x_12 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_processOveriddenDefaultValues(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); lean_dec(x_2); -return x_8; +return x_12; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getNestedProjectionArg___boxed(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_panic___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___spec__1___closed__1() { _start: { -lean_object* x_7; -x_7 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getNestedProjectionArg(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_object* x_1; +x_1 = l_Lean_Elab_Term_instInhabitedTermElabM(lean_box(0)); +return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___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_panic___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___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_8; lean_object* x_9; -x_8 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_8, 0, x_1); -x_9 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_9, 0, x_8); -lean_ctor_set(x_9, 1, x_7); -return x_9; +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = l_panic___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___spec__1___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; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__1() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___spec__2___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("invalid projection name ", 24, 24); +x_1 = lean_mk_string_unchecked("failed to copy fields from parent structure", 43, 43); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__2() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___spec__2___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__1; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___spec__2___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3() { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___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_1; lean_object* x_2; -x_1 = l_Lean_levelZero; -x_2 = l_Lean_Expr_sort___override(x_1); -return x_2; -} +uint8_t x_14; +x_14 = lean_usize_dec_lt(x_5, x_4); +if (x_14 == 0) +{ +lean_object* x_15; +lean_dec(x_7); +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; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: +else { -lean_object* x_9; -x_9 = l_Lean_Expr_getAppFn(x_3); -if (lean_obj_tag(x_9) == 4) +lean_object* x_16; lean_object* x_17; +x_16 = lean_array_uget(x_3, x_5); +x_17 = l_Lean_RBNode_find___at_Lean_NameMap_find_x3f___spec__1___rarg(x_2, x_16); +lean_dec(x_16); +if (lean_obj_tag(x_17) == 0) { -lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_10 = lean_ctor_get(x_9, 0); -lean_inc(x_10); -lean_dec(x_9); -lean_inc(x_10); -x_11 = l_Lean_getProjectionFnInfo_x3f___at_Lean_Meta_getStuckMVar_x3f___spec__1(x_10, x_4, x_5, x_6, x_7, x_8); -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); -if (lean_obj_tag(x_12) == 0) +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; +lean_dec(x_6); +x_18 = l_Lean_indentExpr(x_1); +x_19 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___spec__2___closed__2; +x_20 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_20, 0, x_19); +lean_ctor_set(x_20, 1, x_18); +x_21 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3; +x_22 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_22, 0, x_20); +lean_ctor_set(x_22, 1, x_21); +x_23 = 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) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; -lean_dec(x_10); -x_13 = lean_ctor_get(x_11, 1); -lean_inc(x_13); -lean_dec(x_11); -x_14 = lean_box(0); -x_15 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__1(x_3, x_14, x_4, x_5, x_6, x_7, x_13); -return x_15; +return x_23; } else { -lean_object* x_16; -x_16 = lean_ctor_get(x_12, 0); -lean_inc(x_16); -lean_dec(x_12); -if (lean_obj_tag(x_10) == 1) +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_23, 0); +x_26 = lean_ctor_get(x_23, 1); +lean_inc(x_26); +lean_inc(x_25); +lean_dec(x_23); +x_27 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +return x_27; +} +} +else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_17 = lean_ctor_get(x_11, 1); -lean_inc(x_17); -lean_dec(x_11); -x_18 = lean_ctor_get(x_16, 1); -lean_inc(x_18); -lean_dec(x_16); -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___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); -x_24 = lean_unsigned_to_nat(1u); -x_25 = lean_nat_sub(x_21, x_24); -lean_dec(x_21); -lean_inc(x_3); -x_26 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_3, x_23, x_25); -x_27 = l_Array_get_x3f___rarg(x_26, x_18); -if (lean_obj_tag(x_27) == 0) +lean_object* x_28; lean_object* x_29; size_t x_30; size_t x_31; +x_28 = lean_ctor_get(x_17, 0); +lean_inc(x_28); +lean_dec(x_17); +x_29 = l_Lean_Expr_app___override(x_6, x_28); +x_30 = 1; +x_31 = lean_usize_add(x_5, x_30); +x_5 = x_31; +x_6 = x_29; +goto _start; +} +} +} +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__1() { +_start: { -lean_object* x_28; lean_object* x_29; -lean_dec(x_26); -lean_dec(x_19); -lean_dec(x_18); -x_28 = lean_box(0); -x_29 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__1(x_3, x_28, x_4, x_5, x_6, x_7, x_17); -return x_29; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean.Elab.Structure", 19, 19); +return x_1; } -else +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__2() { +_start: { -lean_object* x_30; lean_object* x_31; uint8_t x_32; -x_30 = lean_ctor_get(x_27, 0); -lean_inc(x_30); -lean_dec(x_27); -x_31 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getNestedProjectionArg(x_30, x_4, x_5, x_6, x_7, x_17); -x_32 = !lean_is_exclusive(x_31); -if (x_32 == 0) +lean_object* x_1; +x_1 = lean_mk_string_unchecked("_private.Lean.Elab.Structure.0.Lean.Elab.Command.copyNewFieldsFrom.mkCompositeField", 83, 83); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__3() { +_start: { -lean_object* x_33; lean_object* x_34; uint8_t x_35; -x_33 = lean_ctor_get(x_31, 0); -x_34 = lean_ctor_get(x_31, 1); -x_35 = lean_expr_eqv(x_33, x_1); -lean_dec(x_33); -if (x_35 == 0) +lean_object* x_1; +x_1 = lean_mk_string_unchecked("unreachable code has been reached", 33, 33); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__4() { +_start: { -lean_object* x_36; lean_object* x_37; -lean_free_object(x_31); -lean_dec(x_26); -lean_dec(x_19); -lean_dec(x_18); -x_36 = lean_box(0); -x_37 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__1(x_3, x_36, x_4, x_5, x_6, x_7, x_34); -return x_37; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__1; +x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__2; +x_3 = lean_unsigned_to_nat(510u); +x_4 = lean_unsigned_to_nat(68u); +x_5 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__3; +x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); +return x_6; } -else +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField(lean_object* x_1, lean_object* x_2, lean_object* x_3, 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_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_box(0); -x_39 = l_Lean_Name_str___override(x_38, x_19); -x_40 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f(x_2, x_39); -lean_dec(x_39); -if (lean_obj_tag(x_40) == 0) +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_st_ref_get(x_8, x_9); +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_10, 1); +lean_inc(x_12); +lean_dec(x_10); +x_13 = lean_ctor_get(x_11, 0); +lean_inc(x_13); +lean_dec(x_11); +x_14 = l_Lean_Expr_getAppFn(x_1); +if (lean_obj_tag(x_14) == 4) { -lean_object* x_41; lean_object* x_42; -lean_free_object(x_31); -lean_dec(x_26); +lean_object* x_15; lean_object* x_16; 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; size_t x_30; size_t x_31; lean_object* x_32; +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_15); +lean_inc(x_13); +x_17 = l_Lean_getStructureCtor(x_13, x_15); +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_41 = lean_box(0); -x_42 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__1(x_3, x_41, x_4, x_5, x_6, x_7, x_34); -return x_42; -} -else +x_20 = l_Lean_Expr_const___override(x_19, x_16); +x_21 = lean_unsigned_to_nat(0u); +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__4; +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); +lean_inc(x_1); +x_27 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_1, x_24, x_26); +x_28 = l_Lean_mkAppN(x_20, x_27); +lean_dec(x_27); +x_29 = l_Lean_getStructureFields(x_13, x_15); +lean_dec(x_13); +x_30 = lean_array_size(x_29); +x_31 = 0; +x_32 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___spec__2(x_1, x_2, x_29, x_30, x_31, x_28, x_3, x_4, x_5, x_6, x_7, x_8, 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_29); +if (lean_obj_tag(x_32) == 0) { -uint8_t x_43; -lean_dec(x_3); -x_43 = !lean_is_exclusive(x_40); -if (x_43 == 0) +uint8_t x_33; +x_33 = !lean_is_exclusive(x_32); +if (x_33 == 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; -x_44 = lean_ctor_get(x_40, 0); -x_45 = lean_ctor_get(x_44, 2); -lean_inc(x_45); -lean_dec(x_44); -x_46 = lean_nat_add(x_18, x_24); -lean_dec(x_18); -x_47 = lean_array_get_size(x_26); -x_48 = l_Array_toSubarray___rarg(x_26, x_46, x_47); -x_49 = l_Array_ofSubarray___rarg(x_48); -lean_dec(x_48); -x_50 = l_Lean_mkAppN(x_45, x_49); -lean_dec(x_49); -lean_ctor_set_tag(x_40, 0); -lean_ctor_set(x_40, 0, x_50); -lean_ctor_set(x_31, 0, x_40); -return x_31; +return x_32; } else { -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; -x_51 = lean_ctor_get(x_40, 0); -lean_inc(x_51); -lean_dec(x_40); -x_52 = lean_ctor_get(x_51, 2); -lean_inc(x_52); -lean_dec(x_51); -x_53 = lean_nat_add(x_18, x_24); -lean_dec(x_18); -x_54 = lean_array_get_size(x_26); -x_55 = l_Array_toSubarray___rarg(x_26, x_53, x_54); -x_56 = l_Array_ofSubarray___rarg(x_55); -lean_dec(x_55); -x_57 = l_Lean_mkAppN(x_52, x_56); -lean_dec(x_56); -x_58 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_58, 0, x_57); -lean_ctor_set(x_31, 0, x_58); -return x_31; -} -} +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_32, 0); +x_35 = lean_ctor_get(x_32, 1); +lean_inc(x_35); +lean_inc(x_34); +lean_dec(x_32); +x_36 = lean_alloc_ctor(0, 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_59; lean_object* x_60; uint8_t x_61; -x_59 = lean_ctor_get(x_31, 0); -x_60 = lean_ctor_get(x_31, 1); -lean_inc(x_60); -lean_inc(x_59); -lean_dec(x_31); -x_61 = lean_expr_eqv(x_59, x_1); -lean_dec(x_59); -if (x_61 == 0) +uint8_t x_37; +x_37 = !lean_is_exclusive(x_32); +if (x_37 == 0) { -lean_object* x_62; lean_object* x_63; -lean_dec(x_26); -lean_dec(x_19); -lean_dec(x_18); -x_62 = lean_box(0); -x_63 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__1(x_3, x_62, x_4, x_5, x_6, x_7, x_60); -return x_63; +return x_32; } else { -lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_64 = lean_box(0); -x_65 = l_Lean_Name_str___override(x_64, x_19); -x_66 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f(x_2, x_65); -lean_dec(x_65); -if (lean_obj_tag(x_66) == 0) -{ -lean_object* x_67; lean_object* x_68; -lean_dec(x_26); -lean_dec(x_18); -x_67 = lean_box(0); -x_68 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__1(x_3, x_67, x_4, x_5, x_6, x_7, x_60); -return x_68; +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_32, 0); +x_39 = lean_ctor_get(x_32, 1); +lean_inc(x_39); +lean_inc(x_38); +lean_dec(x_32); +x_40 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +return x_40; +} +} } else { -lean_object* x_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_dec(x_3); -x_69 = lean_ctor_get(x_66, 0); -lean_inc(x_69); -if (lean_is_exclusive(x_66)) { - lean_ctor_release(x_66, 0); - x_70 = x_66; -} else { - lean_dec_ref(x_66); - x_70 = lean_box(0); +lean_object* x_41; lean_object* x_42; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_1); +x_41 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__4; +x_42 = l_panic___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___spec__1(x_41, x_3, x_4, x_5, x_6, x_7, x_8, x_12); +return x_42; } -x_71 = lean_ctor_get(x_69, 2); -lean_inc(x_71); -lean_dec(x_69); -x_72 = lean_nat_add(x_18, x_24); -lean_dec(x_18); -x_73 = lean_array_get_size(x_26); -x_74 = l_Array_toSubarray___rarg(x_26, x_72, x_73); -x_75 = l_Array_ofSubarray___rarg(x_74); -lean_dec(x_74); -x_76 = l_Lean_mkAppN(x_71, x_75); -lean_dec(x_75); -if (lean_is_scalar(x_70)) { - x_77 = lean_alloc_ctor(0, 1, 0); -} else { - x_77 = x_70; - lean_ctor_set_tag(x_77, 0); } -lean_ctor_set(x_77, 0, x_76); -x_78 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_78, 0, x_77); -lean_ctor_set(x_78, 1, x_60); -return x_78; } +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +size_t x_14; size_t x_15; lean_object* x_16; +x_14 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_15 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_16 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___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_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_3); +lean_dec(x_2); +return x_16; } } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField(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; } } -else -{ -uint8_t x_79; -lean_dec(x_16); -lean_dec(x_3); -x_79 = !lean_is_exclusive(x_11); -if (x_79 == 0) +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields___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_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_80 = lean_ctor_get(x_11, 1); -x_81 = lean_ctor_get(x_11, 0); -lean_dec(x_81); -x_82 = l_Lean_MessageData_ofName(x_10); -x_83 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__2; -lean_ctor_set_tag(x_11, 7); -lean_ctor_set(x_11, 1, x_82); -lean_ctor_set(x_11, 0, x_83); -x_84 = l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__4; -x_85 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_85, 0, x_11); -lean_ctor_set(x_85, 1, x_84); -x_86 = l_Lean_throwError___at_Lean_Meta_mkSimpCongrTheorem___spec__4(x_85, x_4, x_5, x_6, x_7, x_80); -x_87 = !lean_is_exclusive(x_86); -if (x_87 == 0) +lean_object* x_13; +x_13 = l_Lean_Meta_getStructureName(x_4, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_13) == 0) { -return x_86; +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_13, 1); +lean_inc(x_15); +lean_dec(x_13); +x_16 = lean_st_ref_get(x_11, x_15); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +x_19 = lean_ctor_get(x_17, 0); +lean_inc(x_19); +lean_dec(x_17); +lean_inc(x_14); +x_20 = l_Lean_getStructureFields(x_19, x_14); +lean_dec(x_19); +x_21 = lean_box(0); +x_22 = lean_unsigned_to_nat(0u); +x_23 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg(x_1, x_4, x_5, x_14, x_20, x_22, x_2, x_21, x_3, x_6, x_7, x_8, x_9, x_10, x_11, x_18); +return x_23; } else { -lean_object* x_88; lean_object* x_89; lean_object* x_90; -x_88 = lean_ctor_get(x_86, 0); -x_89 = lean_ctor_get(x_86, 1); -lean_inc(x_89); -lean_inc(x_88); -lean_dec(x_86); -x_90 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_90, 0, x_88); -lean_ctor_set(x_90, 1, x_89); -return x_90; -} +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_5); +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) +{ +return x_13; } 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_11, 1); -lean_inc(x_91); -lean_dec(x_11); -x_92 = l_Lean_MessageData_ofName(x_10); -x_93 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__2; -x_94 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_94, 0, x_93); -lean_ctor_set(x_94, 1, x_92); -x_95 = l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__4; -x_96 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_96, 0, x_94); -lean_ctor_set(x_96, 1, x_95); -x_97 = l_Lean_throwError___at_Lean_Meta_mkSimpCongrTheorem___spec__4(x_96, x_4, x_5, x_6, x_7, x_91); -x_98 = lean_ctor_get(x_97, 0); -lean_inc(x_98); -x_99 = lean_ctor_get(x_97, 1); -lean_inc(x_99); -if (lean_is_exclusive(x_97)) { - lean_ctor_release(x_97, 0); - lean_ctor_release(x_97, 1); - x_100 = x_97; -} else { - lean_dec_ref(x_97); - x_100 = lean_box(0); -} -if (lean_is_scalar(x_100)) { - x_101 = lean_alloc_ctor(1, 2, 0); -} else { - x_101 = x_100; -} -lean_ctor_set(x_101, 0, x_98); -lean_ctor_set(x_101, 1, x_99); -return x_101; +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; } } } } -else +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields(lean_object* x_1) { +_start: { -lean_object* x_102; lean_object* x_103; -lean_dec(x_9); -x_102 = lean_box(0); -x_103 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__1(x_3, x_102, x_4, x_5, x_6, x_7, x_8); -return x_103; -} +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields___rarg), 12, 0); +return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__3___closed__1() { +LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___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; -x_1 = lean_box(0); -x_2 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = l_panic___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___spec__1___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_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___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_panic___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___spec__1(lean_object* x_1) { _start: { -lean_object* x_7; lean_object* x_8; -x_7 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__3___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); -return x_8; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_panic___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___spec__1___rarg), 8, 0); +return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19) { _start: { -lean_object* x_10; uint8_t x_11; -x_10 = lean_st_ref_get(x_8, x_9); -x_11 = !lean_is_exclusive(x_10); -if (x_11 == 0) -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_12 = lean_ctor_get(x_10, 0); -x_13 = lean_ctor_get(x_10, 1); -x_14 = lean_ctor_get(x_12, 0); -lean_inc(x_14); -lean_dec(x_12); -x_15 = l_Lean_Meta_getStructureName(x_1, x_5, x_6, x_7, x_8, x_13); -if (lean_obj_tag(x_15) == 0) +lean_object* x_20; lean_object* x_21; +lean_inc(x_12); +lean_inc(x_2); +x_20 = l_Lean_RBNode_insert___at_Lean_NameMap_insert___spec__1___rarg(x_1, x_2, x_12); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_13); +lean_inc(x_2); +lean_inc(x_4); +lean_inc(x_3); +x_21 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f(x_20, x_3, x_4, x_2, x_13, x_14, x_15, x_16, x_17, x_18, x_19); +if (lean_obj_tag(x_21) == 0) { -uint8_t x_16; -x_16 = !lean_is_exclusive(x_15); -if (x_16 == 0) +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; lean_object* x_29; +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_2); +lean_inc(x_5); +x_24 = l_Lean_Name_append(x_5, x_2); +lean_inc(x_6); +x_25 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_toVisibility(x_6, x_17, x_18, x_23); +x_26 = lean_ctor_get(x_25, 0); +lean_inc(x_26); +x_27 = lean_ctor_get(x_25, 1); +lean_inc(x_27); +lean_dec(x_25); +x_28 = lean_unbox(x_26); +lean_dec(x_26); +lean_inc(x_13); +x_29 = l_Lean_Elab_applyVisibility___at_Lean_Elab_Term_expandDeclId___spec__5(x_28, x_24, x_13, x_14, x_15, x_16, x_17, x_18, x_27); +if (lean_obj_tag(x_29) == 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); -x_19 = l_Lean_getFieldInfo_x3f(x_14, x_17, x_3); -lean_dec(x_14); -if (lean_obj_tag(x_19) == 0) -{ -lean_free_object(x_10); -lean_dec(x_8); -lean_dec(x_7); +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_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_30 = lean_ctor_get(x_29, 0); +lean_inc(x_30); +x_31 = lean_ctor_get(x_29, 1); +lean_inc(x_31); +lean_dec(x_29); +x_32 = lean_st_ref_get(x_18, 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); +lean_dec(x_32); +x_35 = lean_ctor_get(x_33, 0); +lean_inc(x_35); +lean_dec(x_33); +x_36 = lean_ctor_get(x_6, 1); +lean_inc(x_36); lean_dec(x_6); -lean_dec(x_5); -lean_ctor_set(x_15, 0, x_2); -return x_15; +x_37 = lean_ctor_get(x_17, 5); +lean_inc(x_37); +x_38 = 1; +x_39 = l_Lean_findDocString_x3f(x_35, x_36, x_38, x_34); +lean_dec(x_35); +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_13); +lean_inc(x_30); +x_42 = l_Lean_addDocString_x27___at_Lean_Elab_Term_expandDeclId___spec__8(x_30, x_40, x_13, x_14, x_15, x_16, x_17, x_18, x_41); +if (lean_obj_tag(x_42) == 0) +{ +lean_object* x_43; uint8_t x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_43 = lean_ctor_get(x_42, 1); +lean_inc(x_43); +lean_dec(x_42); +x_44 = 1; +x_45 = lean_alloc_ctor(0, 5, 1); +lean_ctor_set(x_45, 0, x_37); +lean_ctor_set(x_45, 1, x_2); +lean_ctor_set(x_45, 2, x_30); +lean_ctor_set(x_45, 3, x_12); +lean_ctor_set(x_45, 4, x_22); +lean_ctor_set_uint8(x_45, sizeof(void*)*5, x_44); +x_46 = lean_array_push(x_7, x_45); +x_47 = lean_unsigned_to_nat(1u); +x_48 = lean_nat_add(x_8, x_47); +x_49 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg(x_5, x_9, x_10, x_4, x_11, x_48, x_46, x_20, x_3, x_13, x_14, x_15, x_16, x_17, x_18, x_43); +return x_49; } else { -lean_object* x_20; lean_object* x_21; -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); -lean_dec(x_19); -x_21 = lean_ctor_get(x_20, 3); -lean_inc(x_21); +uint8_t x_50; +lean_dec(x_37); +lean_dec(x_30); +lean_dec(x_22); lean_dec(x_20); -if (lean_obj_tag(x_21) == 0) -{ -lean_free_object(x_10); -lean_dec(x_8); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); lean_dec(x_7); -lean_dec(x_6); lean_dec(x_5); -lean_ctor_set(x_15, 0, x_2); -return x_15; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_50 = !lean_is_exclusive(x_42); +if (x_50 == 0) +{ +return x_42; } 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_free_object(x_15); -x_22 = lean_ctor_get(x_21, 0); -lean_inc(x_22); -lean_dec(x_21); -x_23 = lean_box(0); -lean_ctor_set_tag(x_10, 1); -lean_ctor_set(x_10, 1, x_23); -lean_ctor_set(x_10, 0, x_22); -x_24 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_24, 0, x_2); -lean_ctor_set(x_24, 1, x_10); -x_25 = lean_array_mk(x_24); -x_26 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__12; -x_27 = l_Lean_Meta_mkAppM(x_26, x_25, x_5, x_6, x_7, x_8, x_18); -if (lean_obj_tag(x_27) == 0) +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_28; -x_28 = !lean_is_exclusive(x_27); -if (x_28 == 0) +uint8_t x_54; +lean_dec(x_22); +lean_dec(x_20); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_54 = !lean_is_exclusive(x_29); +if (x_54 == 0) { -return x_27; +return x_29; } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_27, 0); -x_30 = lean_ctor_get(x_27, 1); -lean_inc(x_30); -lean_inc(x_29); -lean_dec(x_27); -x_31 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_31, 0, x_29); -lean_ctor_set(x_31, 1, x_30); -return x_31; +lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_55 = lean_ctor_get(x_29, 0); +x_56 = lean_ctor_get(x_29, 1); +lean_inc(x_56); +lean_inc(x_55); +lean_dec(x_29); +x_57 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_57, 0, x_55); +lean_ctor_set(x_57, 1, x_56); +return x_57; +} } } else { -uint8_t x_32; -x_32 = !lean_is_exclusive(x_27); -if (x_32 == 0) +uint8_t x_58; +lean_dec(x_20); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_58 = !lean_is_exclusive(x_21); +if (x_58 == 0) { -return x_27; +return x_21; } else { -lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_33 = lean_ctor_get(x_27, 0); -x_34 = lean_ctor_get(x_27, 1); -lean_inc(x_34); -lean_inc(x_33); -lean_dec(x_27); -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_59; lean_object* x_60; lean_object* x_61; +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_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); +return x_61; +} } } } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18) { +_start: +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_19 = lean_unsigned_to_nat(1u); +x_20 = lean_nat_add(x_1, x_19); +x_21 = l_Lean_RBNode_insert___at_Lean_NameMap_insert___spec__1___rarg(x_2, x_3, x_4); +x_22 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg(x_5, x_6, x_7, x_8, x_9, x_20, x_11, x_21, x_10, x_12, x_13, x_14, x_15, x_16, x_17, x_18); +return x_22; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___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_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19, lean_object* x_20) { +_start: +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_21 = lean_ctor_get(x_18, 5); +lean_inc(x_21); +lean_inc(x_2); +lean_inc(x_1); +x_22 = l_Lean_Name_append(x_1, x_2); +x_23 = lean_box(0); +x_24 = 3; +lean_inc(x_13); +lean_inc(x_2); +x_25 = lean_alloc_ctor(0, 5, 1); +lean_ctor_set(x_25, 0, x_21); +lean_ctor_set(x_25, 1, x_2); +lean_ctor_set(x_25, 2, x_22); +lean_ctor_set(x_25, 3, x_13); +lean_ctor_set(x_25, 4, x_23); +lean_ctor_set_uint8(x_25, sizeof(void*)*5, x_24); +x_26 = lean_array_push(x_3, x_25); +lean_inc(x_1); +lean_inc(x_13); +x_27 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__2___boxed), 18, 10); +lean_closure_set(x_27, 0, x_4); +lean_closure_set(x_27, 1, x_5); +lean_closure_set(x_27, 2, x_2); +lean_closure_set(x_27, 3, x_13); +lean_closure_set(x_27, 4, x_1); +lean_closure_set(x_27, 5, x_6); +lean_closure_set(x_27, 6, x_7); +lean_closure_set(x_27, 7, x_8); +lean_closure_set(x_27, 8, x_9); +lean_closure_set(x_27, 9, x_10); +x_28 = lean_unsigned_to_nat(0u); +x_29 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg(x_1, x_13, x_11, x_12, x_27, x_28, x_26, x_14, x_15, x_16, x_17, x_18, x_19, x_20); +return x_29; +} } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19) { +_start: +{ +lean_object* x_20; +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +x_20 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField(x_1, x_11, x_13, x_14, x_15, x_16, x_17, x_18, x_19); +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; +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_unsigned_to_nat(1u); +x_24 = lean_nat_add(x_2, x_23); +x_25 = l_Lean_RBNode_insert___at_Lean_NameMap_insert___spec__1___rarg(x_3, x_4, x_21); +x_26 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg(x_5, x_6, x_7, x_8, x_9, x_24, x_10, x_25, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_22); +return x_26; } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_15, 0); -x_37 = lean_ctor_get(x_15, 1); -lean_inc(x_37); -lean_inc(x_36); +uint8_t x_27; +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); lean_dec(x_15); -x_38 = l_Lean_getFieldInfo_x3f(x_14, x_36, x_3); lean_dec(x_14); -if (lean_obj_tag(x_38) == 0) -{ -lean_object* x_39; -lean_free_object(x_10); +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_6); lean_dec(x_5); -x_39 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_39, 0, x_2); -lean_ctor_set(x_39, 1, x_37); -return x_39; +lean_dec(x_4); +lean_dec(x_3); +x_27 = !lean_is_exclusive(x_20); +if (x_27 == 0) +{ +return x_20; } else { -lean_object* x_40; lean_object* x_41; -x_40 = lean_ctor_get(x_38, 0); -lean_inc(x_40); -lean_dec(x_38); -x_41 = lean_ctor_get(x_40, 3); -lean_inc(x_41); -lean_dec(x_40); -if (lean_obj_tag(x_41) == 0) +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_20, 0); +x_29 = lean_ctor_get(x_20, 1); +lean_inc(x_29); +lean_inc(x_28); +lean_dec(x_20); +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___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19) { +_start: { -lean_object* x_42; -lean_free_object(x_10); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -x_42 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_42, 0, x_2); -lean_ctor_set(x_42, 1, x_37); -return x_42; +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_20 = lean_unsigned_to_nat(1u); +x_21 = lean_nat_add(x_1, x_20); +x_22 = l_Lean_RBNode_insert___at_Lean_NameMap_insert___spec__1___rarg(x_2, x_3, x_4); +x_23 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg(x_5, x_6, x_7, x_8, x_9, x_21, x_10, x_22, x_11, x_13, x_14, x_15, x_16, x_17, x_18, x_19); +return x_23; } -else +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__1() { +_start: { -lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; -x_43 = lean_ctor_get(x_41, 0); -lean_inc(x_43); -lean_dec(x_41); -x_44 = lean_box(0); -lean_ctor_set_tag(x_10, 1); -lean_ctor_set(x_10, 1, x_44); -lean_ctor_set(x_10, 0, x_43); -x_45 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_45, 0, x_2); -lean_ctor_set(x_45, 1, x_10); -x_46 = lean_array_mk(x_45); -x_47 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__12; -x_48 = l_Lean_Meta_mkAppM(x_47, x_46, x_5, x_6, x_7, x_8, x_37); -if (lean_obj_tag(x_48) == 0) +lean_object* x_1; +x_1 = lean_mk_string_unchecked("_private.Lean.Elab.Structure.0.Lean.Elab.Command.copyNewFieldsFrom.copyFields.copy", 82, 82); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__2() { +_start: { -lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_49 = lean_ctor_get(x_48, 0); -lean_inc(x_49); -x_50 = lean_ctor_get(x_48, 1); -lean_inc(x_50); -if (lean_is_exclusive(x_48)) { - lean_ctor_release(x_48, 0); - lean_ctor_release(x_48, 1); - x_51 = x_48; -} else { - lean_dec_ref(x_48); - x_51 = lean_box(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___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__1; +x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__1; +x_3 = lean_unsigned_to_nat(466u); +x_4 = lean_unsigned_to_nat(86u); +x_5 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__3; +x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); +return x_6; } -if (lean_is_scalar(x_51)) { - x_52 = lean_alloc_ctor(0, 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; +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("parent field type mismatch, field '", 35, 35); +return x_1; } -else +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__4() { +_start: { -lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; -x_53 = lean_ctor_get(x_48, 0); -lean_inc(x_53); -x_54 = lean_ctor_get(x_48, 1); -lean_inc(x_54); -if (lean_is_exclusive(x_48)) { - lean_ctor_release(x_48, 0); - lean_ctor_release(x_48, 1); - x_55 = x_48; -} else { - lean_dec_ref(x_48); - x_55 = lean_box(0); +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } -if (lean_is_scalar(x_55)) { - x_56 = lean_alloc_ctor(1, 2, 0); -} else { - x_56 = x_55; } -lean_ctor_set(x_56, 0, x_53); -lean_ctor_set(x_56, 1, x_54); -return x_56; +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("' from parent '", 15, 15); +return x_1; +} } +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__5; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__7() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("' ", 2, 2); +return x_1; } } -else +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__8() { +_start: { -uint8_t x_57; -lean_dec(x_14); -lean_free_object(x_10); -lean_dec(x_8); -lean_dec(x_7); +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__7; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +_start: +{ +lean_object* x_17; uint8_t x_18; +x_17 = lean_array_get_size(x_5); +x_18 = lean_nat_dec_lt(x_6, x_17); +lean_dec(x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_dec(x_6); lean_dec(x_5); -lean_dec(x_3); lean_dec(x_2); -x_57 = !lean_is_exclusive(x_15); -if (x_57 == 0) +lean_dec(x_1); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_10); +lean_inc(x_9); +x_19 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_processOveriddenDefaultValues(x_7, x_8, x_9, x_4, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_19) == 0) { -return x_15; +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_19, 1); +lean_inc(x_21); +lean_dec(x_19); +x_22 = lean_apply_10(x_3, x_20, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_21); +return x_22; } else { -lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_58 = lean_ctor_get(x_15, 0); -x_59 = lean_ctor_get(x_15, 1); -lean_inc(x_59); -lean_inc(x_58); +uint8_t x_23; lean_dec(x_15); -x_60 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_60, 0, x_58); -lean_ctor_set(x_60, 1, x_59); -return x_60; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_3); +x_23 = !lean_is_exclusive(x_19); +if (x_23 == 0) +{ +return x_19; +} +else +{ +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_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_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; -x_61 = lean_ctor_get(x_10, 0); -x_62 = lean_ctor_get(x_10, 1); -lean_inc(x_62); -lean_inc(x_61); -lean_dec(x_10); -x_63 = lean_ctor_get(x_61, 0); -lean_inc(x_63); -lean_dec(x_61); -x_64 = l_Lean_Meta_getStructureName(x_1, x_5, x_6, x_7, x_8, x_62); -if (lean_obj_tag(x_64) == 0) +lean_object* x_27; lean_object* x_28; +x_27 = lean_array_fget(x_5, x_6); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_27); +lean_inc(x_2); +lean_inc(x_7); +x_28 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType(x_7, x_2, x_27, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_28) == 0) { -lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_65 = lean_ctor_get(x_64, 0); -lean_inc(x_65); -x_66 = lean_ctor_get(x_64, 1); -lean_inc(x_66); -if (lean_is_exclusive(x_64)) { - lean_ctor_release(x_64, 0); - lean_ctor_release(x_64, 1); - x_67 = x_64; -} else { - lean_dec_ref(x_64); - x_67 = lean_box(0); -} -x_68 = l_Lean_getFieldInfo_x3f(x_63, x_65, x_3); -lean_dec(x_63); -if (lean_obj_tag(x_68) == 0) +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_28, 0); +lean_inc(x_29); +x_30 = lean_ctor_get(x_28, 1); +lean_inc(x_30); +lean_dec(x_28); +x_31 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f(x_7, x_27); +if (lean_obj_tag(x_31) == 0) { -lean_object* x_69; +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_32 = lean_st_ref_get(x_15, x_30); +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_dec(x_33); +lean_inc(x_27); +lean_inc(x_4); +x_36 = l_Lean_getFieldInfo_x3f(x_35, x_4, x_27); +lean_dec(x_35); +if (lean_obj_tag(x_36) == 0) +{ +lean_object* x_37; lean_object* x_38; +lean_dec(x_29); +lean_dec(x_27); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -if (lean_is_scalar(x_67)) { - x_69 = lean_alloc_ctor(0, 2, 0); -} else { - x_69 = x_67; -} -lean_ctor_set(x_69, 0, x_2); -lean_ctor_set(x_69, 1, x_66); -return x_69; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_37 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__2; +x_38 = l_panic___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___spec__1___rarg(x_37, x_10, x_11, x_12, x_13, x_14, x_15, x_34); +return x_38; } else { -lean_object* x_70; lean_object* x_71; -x_70 = lean_ctor_get(x_68, 0); -lean_inc(x_70); -lean_dec(x_68); -x_71 = lean_ctor_get(x_70, 3); -lean_inc(x_71); -lean_dec(x_70); -if (lean_obj_tag(x_71) == 0) +lean_object* x_39; lean_object* x_40; +x_39 = lean_ctor_get(x_36, 0); +lean_inc(x_39); +lean_dec(x_36); +x_40 = lean_ctor_get(x_39, 2); +lean_inc(x_40); +if (lean_obj_tag(x_40) == 0) { -lean_object* x_72; -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -if (lean_is_scalar(x_67)) { - x_72 = lean_alloc_ctor(0, 2, 0); -} else { - x_72 = x_67; -} -lean_ctor_set(x_72, 0, x_2); -lean_ctor_set(x_72, 1, x_66); -return x_72; +uint8_t x_41; lean_object* x_42; uint8_t x_43; lean_object* x_44; +x_41 = lean_ctor_get_uint8(x_39, sizeof(void*)*4); +lean_inc(x_27); +x_42 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__1___boxed), 19, 11); +lean_closure_set(x_42, 0, x_8); +lean_closure_set(x_42, 1, x_27); +lean_closure_set(x_42, 2, x_9); +lean_closure_set(x_42, 3, x_4); +lean_closure_set(x_42, 4, x_1); +lean_closure_set(x_42, 5, x_39); +lean_closure_set(x_42, 6, x_7); +lean_closure_set(x_42, 7, x_6); +lean_closure_set(x_42, 8, x_2); +lean_closure_set(x_42, 9, x_3); +lean_closure_set(x_42, 10, x_5); +x_43 = 0; +x_44 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__1___rarg(x_27, x_41, x_29, x_42, x_43, x_10, x_11, x_12, x_13, x_14, x_15, x_34); +return x_44; } 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_dec(x_67); -x_73 = lean_ctor_get(x_71, 0); -lean_inc(x_73); -lean_dec(x_71); -x_74 = lean_box(0); -x_75 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_75, 0, x_73); -lean_ctor_set(x_75, 1, x_74); -x_76 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_76, 0, x_2); -lean_ctor_set(x_76, 1, x_75); -x_77 = lean_array_mk(x_76); -x_78 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__12; -x_79 = l_Lean_Meta_mkAppM(x_78, x_77, x_5, x_6, x_7, x_8, x_66); -if (lean_obj_tag(x_79) == 0) +uint8_t x_45; lean_object* x_46; +lean_dec(x_40); +x_45 = lean_ctor_get_uint8(x_39, sizeof(void*)*4); +x_46 = l_Lean_Meta_getStructureName(x_29, x_12, x_13, x_14, x_15, x_34); +if (lean_obj_tag(x_46) == 0) { -lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; -x_80 = lean_ctor_get(x_79, 0); -lean_inc(x_80); -x_81 = lean_ctor_get(x_79, 1); -lean_inc(x_81); -if (lean_is_exclusive(x_79)) { - lean_ctor_release(x_79, 0); - lean_ctor_release(x_79, 1); - x_82 = x_79; -} else { - lean_dec_ref(x_79); - x_82 = lean_box(0); -} -if (lean_is_scalar(x_82)) { - x_83 = lean_alloc_ctor(0, 2, 0); -} else { - x_83 = x_82; -} -lean_ctor_set(x_83, 0, x_80); -lean_ctor_set(x_83, 1, x_81); -return x_83; +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_47 = lean_ctor_get(x_46, 0); +lean_inc(x_47); +x_48 = lean_ctor_get(x_46, 1); +lean_inc(x_48); +lean_dec(x_46); +lean_inc(x_47); +x_49 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f(x_7, x_47, x_14, x_15, x_48); +x_50 = lean_ctor_get(x_49, 0); +lean_inc(x_50); +if (lean_obj_tag(x_50) == 0) +{ +lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; uint8_t x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; uint8_t x_60; lean_object* x_61; +lean_dec(x_27); +x_51 = lean_ctor_get(x_49, 1); +lean_inc(x_51); +lean_dec(x_49); +x_52 = lean_st_ref_get(x_15, x_51); +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_ctor_get(x_53, 0); +lean_inc(x_55); +lean_dec(x_53); +x_56 = 1; +lean_inc(x_47); +x_57 = l_Lean_getStructureFieldsFlattened(x_55, x_47, x_56); +lean_dec(x_55); +x_58 = lean_ctor_get(x_39, 0); +lean_inc(x_58); +lean_dec(x_39); +lean_inc(x_58); +x_59 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__3___boxed), 20, 12); +lean_closure_set(x_59, 0, x_1); +lean_closure_set(x_59, 1, x_58); +lean_closure_set(x_59, 2, x_7); +lean_closure_set(x_59, 3, x_6); +lean_closure_set(x_59, 4, x_8); +lean_closure_set(x_59, 5, x_2); +lean_closure_set(x_59, 6, x_3); +lean_closure_set(x_59, 7, x_4); +lean_closure_set(x_59, 8, x_5); +lean_closure_set(x_59, 9, x_9); +lean_closure_set(x_59, 10, x_47); +lean_closure_set(x_59, 11, x_57); +x_60 = 0; +x_61 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__1___rarg(x_58, x_45, x_29, x_59, x_60, x_10, x_11, x_12, x_13, x_14, x_15, x_54); +return x_61; } else { -lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; -x_84 = lean_ctor_get(x_79, 0); -lean_inc(x_84); -x_85 = lean_ctor_get(x_79, 1); -lean_inc(x_85); -if (lean_is_exclusive(x_79)) { - lean_ctor_release(x_79, 0); - lean_ctor_release(x_79, 1); - x_86 = x_79; -} else { - lean_dec_ref(x_79); - x_86 = lean_box(0); -} -if (lean_is_scalar(x_86)) { - x_87 = lean_alloc_ctor(1, 2, 0); -} else { - x_87 = x_86; -} -lean_ctor_set(x_87, 0, x_84); -lean_ctor_set(x_87, 1, x_85); -return x_87; -} -} +lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; +lean_dec(x_50); +lean_dec(x_39); +x_62 = lean_ctor_get(x_49, 1); +lean_inc(x_62); +lean_dec(x_49); +x_63 = lean_box(0); +x_64 = l_Lean_RBNode_insert___at_Lean_NameSet_insert___spec__1(x_9, x_47, x_63); +lean_inc(x_1); +lean_inc(x_29); +x_65 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__4___boxed), 19, 9); +lean_closure_set(x_65, 0, x_29); +lean_closure_set(x_65, 1, x_6); +lean_closure_set(x_65, 2, x_8); +lean_closure_set(x_65, 3, x_27); +lean_closure_set(x_65, 4, x_1); +lean_closure_set(x_65, 5, x_2); +lean_closure_set(x_65, 6, x_3); +lean_closure_set(x_65, 7, x_4); +lean_closure_set(x_65, 8, x_5); +x_66 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields___rarg(x_1, x_7, x_64, x_29, x_65, x_10, x_11, x_12, x_13, x_14, x_15, x_62); +return x_66; } } else { -lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; -lean_dec(x_63); +uint8_t x_67; +lean_dec(x_39); +lean_dec(x_29); +lean_dec(x_27); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_88 = lean_ctor_get(x_64, 0); -lean_inc(x_88); -x_89 = lean_ctor_get(x_64, 1); -lean_inc(x_89); -if (lean_is_exclusive(x_64)) { - lean_ctor_release(x_64, 0); - lean_ctor_release(x_64, 1); - x_90 = x_64; -} else { - lean_dec_ref(x_64); - x_90 = lean_box(0); -} -if (lean_is_scalar(x_90)) { - x_91 = lean_alloc_ctor(1, 2, 0); -} else { - x_91 = x_90; -} -lean_ctor_set(x_91, 0, x_88); -lean_ctor_set(x_91, 1, x_89); -return x_91; -} -} -} -} -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___closed__1() { -_start: +lean_dec(x_1); +x_67 = !lean_is_exclusive(x_46); +if (x_67 == 0) { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__3___boxed), 6, 0); -return x_1; -} +return x_46; } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___closed__2() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("unsupported dependent field in ", 31, 31); -return x_1; -} +lean_object* x_68; lean_object* x_69; lean_object* x_70; +x_68 = lean_ctor_get(x_46, 0); +x_69 = lean_ctor_get(x_46, 1); +lean_inc(x_69); +lean_inc(x_68); +lean_dec(x_46); +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; } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___closed__2; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked(" : ", 3, 3); -return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___closed__5() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___closed__4; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_1); -lean_inc(x_4); -x_10 = l_Lean_Meta_mkProjection(x_4, x_1, 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_object* x_71; lean_object* x_72; lean_object* x_73; +x_71 = lean_ctor_get(x_31, 0); +lean_inc(x_71); +lean_dec(x_31); +x_72 = lean_ctor_get(x_71, 3); +lean_inc(x_72); +lean_dec(x_71); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); lean_inc(x_12); -lean_dec(x_10); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -x_13 = lean_infer_type(x_11, x_5, x_6, x_7, x_8, x_12); -if (lean_obj_tag(x_13) == 0) +lean_inc(x_72); +x_73 = lean_infer_type(x_72, x_12, x_13, x_14, x_15, x_30); +if (lean_obj_tag(x_73) == 0) { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; -x_14 = lean_ctor_get(x_13, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_13, 1); +lean_object* x_74; lean_object* x_75; lean_object* 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); lean_inc(x_15); -lean_dec(x_13); -lean_inc(x_4); -x_16 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___boxed), 8, 2); -lean_closure_set(x_16, 0, x_4); -lean_closure_set(x_16, 1, x_2); -x_17 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___closed__1; -x_18 = 0; -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -x_19 = l_Lean_Meta_transform___at_Lean_Meta_zetaReduce___spec__1(x_14, x_17, x_16, x_18, x_18, x_5, x_6, x_7, x_8, x_15); -if (lean_obj_tag(x_19) == 0) -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; -x_20 = lean_ctor_get(x_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_Expr_fvarId_x21(x_4); -lean_dec(x_4); -x_23 = l_Lean_Expr_hasAnyFVar_visit___at_Lean_Expr_containsFVar___spec__1(x_22, x_20); -lean_dec(x_22); -if (x_23 == 0) +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_74); +lean_inc(x_29); +x_76 = l_Lean_Meta_isExprDefEq(x_29, x_74, x_12, x_13, x_14, x_15, x_75); +if (lean_obj_tag(x_76) == 0) { -lean_object* x_24; lean_object* x_25; -x_24 = lean_box(0); -x_25 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__4(x_3, x_20, x_1, x_24, x_5, x_6, x_7, x_8, x_21); -return x_25; -} -else +lean_object* x_77; uint8_t x_78; +x_77 = lean_ctor_get(x_76, 0); +lean_inc(x_77); +x_78 = lean_unbox(x_77); +lean_dec(x_77); +if (x_78 == 0) { -lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; -x_26 = l_Lean_MessageData_ofName(x_1); -x_27 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___closed__3; -x_28 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_28, 0, x_27); -lean_ctor_set(x_28, 1, x_26); -x_29 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___closed__5; -x_30 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_30, 0, x_28); -lean_ctor_set(x_30, 1, x_29); -x_31 = l_Lean_MessageData_ofExpr(x_20); -x_32 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_32, 0, x_30); -lean_ctor_set(x_32, 1, x_31); -x_33 = l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__4; -x_34 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_34, 0, x_32); -lean_ctor_set(x_34, 1, x_33); -x_35 = l_Lean_throwError___at_Lean_Meta_mkSimpCongrTheorem___spec__4(x_34, x_5, x_6, x_7, x_8, x_21); +lean_object* x_79; lean_object* x_80; +lean_dec(x_72); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -x_36 = !lean_is_exclusive(x_35); -if (x_36 == 0) +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_79 = lean_ctor_get(x_76, 1); +lean_inc(x_79); +lean_dec(x_76); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +x_80 = l_Lean_Meta_mkHasTypeButIsExpectedMsg(x_29, x_74, x_12, x_13, x_14, x_15, x_79); +if (lean_obj_tag(x_80) == 0) { -return x_35; +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; uint8_t x_96; +x_81 = lean_ctor_get(x_80, 0); +lean_inc(x_81); +x_82 = lean_ctor_get(x_80, 1); +lean_inc(x_82); +lean_dec(x_80); +x_83 = l_Lean_MessageData_ofName(x_27); +x_84 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__4; +x_85 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_85, 0, x_84); +lean_ctor_set(x_85, 1, x_83); +x_86 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__6; +x_87 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_87, 0, x_85); +lean_ctor_set(x_87, 1, x_86); +x_88 = l_Lean_MessageData_ofName(x_4); +x_89 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_89, 0, x_87); +lean_ctor_set(x_89, 1, x_88); +x_90 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__8; +x_91 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_91, 0, x_89); +lean_ctor_set(x_91, 1, x_90); +x_92 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_92, 0, x_91); +lean_ctor_set(x_92, 1, x_81); +x_93 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3; +x_94 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_94, 0, x_92); +lean_ctor_set(x_94, 1, x_93); +x_95 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_94, x_10, x_11, x_12, x_13, x_14, x_15, x_82); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +x_96 = !lean_is_exclusive(x_95); +if (x_96 == 0) +{ +return x_95; } 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_97; lean_object* x_98; lean_object* x_99; +x_97 = lean_ctor_get(x_95, 0); +x_98 = lean_ctor_get(x_95, 1); +lean_inc(x_98); +lean_inc(x_97); +lean_dec(x_95); +x_99 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_99, 0, x_97); +lean_ctor_set(x_99, 1, x_98); +return x_99; } } else { -uint8_t x_40; -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); +uint8_t x_100; +lean_dec(x_27); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); lean_dec(x_4); -lean_dec(x_1); -x_40 = !lean_is_exclusive(x_19); -if (x_40 == 0) +x_100 = !lean_is_exclusive(x_80); +if (x_100 == 0) { -return x_19; +return x_80; } else { -lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_ctor_get(x_19, 0); -x_42 = lean_ctor_get(x_19, 1); -lean_inc(x_42); -lean_inc(x_41); -lean_dec(x_19); -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_101; lean_object* x_102; lean_object* x_103; +x_101 = lean_ctor_get(x_80, 0); +x_102 = lean_ctor_get(x_80, 1); +lean_inc(x_102); +lean_inc(x_101); +lean_dec(x_80); +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 { -uint8_t x_44; +lean_object* x_104; lean_object* x_105; lean_object* x_106; +lean_dec(x_74); +lean_dec(x_29); +x_104 = lean_ctor_get(x_76, 1); +lean_inc(x_104); +lean_dec(x_76); +x_105 = lean_box(0); +x_106 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__5(x_6, x_8, x_27, x_72, x_1, x_2, x_3, x_4, x_5, x_7, x_9, x_105, x_10, x_11, x_12, x_13, x_14, x_15, x_104); +lean_dec(x_6); +return x_106; +} +} +else +{ +uint8_t x_107; +lean_dec(x_74); +lean_dec(x_72); +lean_dec(x_29); +lean_dec(x_27); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_44 = !lean_is_exclusive(x_13); -if (x_44 == 0) +x_107 = !lean_is_exclusive(x_76); +if (x_107 == 0) { -return x_13; +return x_76; } else { -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_13, 0); -x_46 = lean_ctor_get(x_13, 1); -lean_inc(x_46); -lean_inc(x_45); -lean_dec(x_13); -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_108; lean_object* x_109; lean_object* x_110; +x_108 = lean_ctor_get(x_76, 0); +x_109 = lean_ctor_get(x_76, 1); +lean_inc(x_109); +lean_inc(x_108); +lean_dec(x_76); +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_48; +uint8_t x_111; +lean_dec(x_72); +lean_dec(x_29); +lean_dec(x_27); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_48 = !lean_is_exclusive(x_10); -if (x_48 == 0) +x_111 = !lean_is_exclusive(x_73); +if (x_111 == 0) { -return x_10; +return x_73; } else { -lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_49 = lean_ctor_get(x_10, 0); -x_50 = lean_ctor_get(x_10, 1); -lean_inc(x_50); -lean_inc(x_49); -lean_dec(x_10); -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_112; lean_object* x_113; lean_object* x_114; +x_112 = lean_ctor_get(x_73, 0); +x_113 = lean_ctor_get(x_73, 1); +lean_inc(x_113); +lean_inc(x_112); +lean_dec(x_73); +x_114 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_114, 0, x_112); +lean_ctor_set(x_114, 1, x_113); +return x_114; } } } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType(lean_object* x_1, lean_object* x_2, lean_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; uint8_t x_14; lean_object* x_15; -x_9 = l_Lean_mkFreshId___at_Lean_Meta_mkFreshExprMVarAt___spec__2___rarg(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); +uint8_t x_115; +lean_dec(x_27); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); lean_dec(x_9); -lean_inc(x_2); -x_12 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___boxed), 9, 3); -lean_closure_set(x_12, 0, x_3); -lean_closure_set(x_12, 1, x_1); -lean_closure_set(x_12, 2, x_2); -x_13 = 0; -x_14 = 0; -x_15 = l_Lean_Meta_withLocalDecl___at_Lean_Meta_GeneralizeTelescope_generalizeTelescopeAux___spec__1___rarg(x_10, x_13, x_2, x_12, x_14, x_4, x_5, x_6, x_7, x_11); -return x_15; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__1___boxed(lean_object* x_1, 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_Structure_0__Lean_Elab_Command_getFieldType___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_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); +x_115 = !lean_is_exclusive(x_28); +if (x_115 == 0) +{ +return x_28; +} +else +{ +lean_object* x_116; lean_object* x_117; lean_object* x_118; +x_116 = lean_ctor_get(x_28, 0); +x_117 = lean_ctor_get(x_28, 1); +lean_inc(x_117); +lean_inc(x_116); +lean_dec(x_28); +x_118 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_118, 0, x_116); +lean_ctor_set(x_118, 1, x_117); +return x_118; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___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___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy(lean_object* x_1) { _start: { -lean_object* x_9; -x_9 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -return x_9; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg), 16, 0); +return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___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___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___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_7; -x_7 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_7; +lean_object* x_20; +x_20 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19); +lean_dec(x_8); +return x_20; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___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]; +lean_object* x_18 = _args[17]; _start: { -lean_object* x_10; -x_10 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_4); +lean_object* x_19; +x_19 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18); lean_dec(x_1); -return x_10; +return x_19; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___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]; +lean_object* x_18 = _args[17]; +lean_object* x_19 = _args[18]; +lean_object* x_20 = _args[19]; _start: { -lean_object* x_10; -x_10 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_3); -return x_10; +lean_object* x_21; +x_21 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20); +return x_21; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_toVisibility___closed__1() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__4___boxed(lean_object** _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_1; -x_1 = l_Lean_protectedExt; -return x_1; +lean_object* x_20; +x_20 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19); +lean_dec(x_11); +lean_dec(x_2); +return x_20; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_toVisibility(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___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]; +lean_object* x_18 = _args[17]; +lean_object* x_19 = _args[18]; _start: { -lean_object* x_5; uint8_t x_6; -x_5 = lean_st_ref_get(x_3, x_4); -x_6 = !lean_is_exclusive(x_5); -if (x_6 == 0) -{ -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; -x_7 = lean_ctor_get(x_5, 0); -x_8 = lean_ctor_get(x_7, 0); -lean_inc(x_8); -lean_dec(x_7); -x_9 = lean_ctor_get(x_1, 1); -lean_inc(x_9); +lean_object* x_20; +x_20 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19); +lean_dec(x_12); lean_dec(x_1); -x_10 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_toVisibility___closed__1; -lean_inc(x_9); -x_11 = l_Lean_TagDeclarationExtension_isTagged(x_10, x_8, x_9); -lean_dec(x_8); -if (x_11 == 0) -{ -uint8_t x_12; -x_12 = l_Lean_isPrivateName(x_9); -lean_dec(x_9); -if (x_12 == 0) -{ -uint8_t x_13; lean_object* x_14; -x_13 = 0; -x_14 = lean_box(x_13); -lean_ctor_set(x_5, 0, x_14); -return x_5; +return x_20; } -else +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom___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) { +_start: { -uint8_t x_15; lean_object* x_16; -x_15 = 2; -x_16 = lean_box(x_15); -lean_ctor_set(x_5, 0, x_16); -return x_5; +lean_object* x_12; +x_12 = lean_apply_8(x_1, x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_12; } } -else +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom___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: { -uint8_t x_17; lean_object* x_18; -lean_dec(x_9); -x_17 = 1; -x_18 = lean_box(x_17); -lean_ctor_set(x_5, 0, x_18); -return x_5; +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom___rarg___lambda__1___boxed), 11, 1); +lean_closure_set(x_12, 0, x_4); +x_13 = l_Lean_NameSet_empty; +x_14 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields___rarg(x_1, x_2, x_13, x_3, x_12, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_14; } } -else -{ -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_5, 0); -x_20 = lean_ctor_get(x_5, 1); -lean_inc(x_20); -lean_inc(x_19); -lean_dec(x_5); -x_21 = lean_ctor_get(x_19, 0); -lean_inc(x_21); -lean_dec(x_19); -x_22 = lean_ctor_get(x_1, 1); -lean_inc(x_22); -lean_dec(x_1); -x_23 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_toVisibility___closed__1; -lean_inc(x_22); -x_24 = l_Lean_TagDeclarationExtension_isTagged(x_23, x_21, x_22); -lean_dec(x_21); -if (x_24 == 0) -{ -uint8_t x_25; -x_25 = l_Lean_isPrivateName(x_22); -lean_dec(x_22); -if (x_25 == 0) +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom(lean_object* x_1) { +_start: { -uint8_t x_26; lean_object* x_27; lean_object* x_28; -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_20); -return x_28; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom___rarg), 11, 0); +return x_2; } -else +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: { -uint8_t x_29; lean_object* x_30; lean_object* x_31; -x_29 = 2; -x_30 = lean_box(x_29); -x_31 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_31, 0, x_30); -lean_ctor_set(x_31, 1, x_20); -return x_31; +lean_object* x_12; +x_12 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_4); +lean_dec(x_3); +return x_12; } } -else +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkToParentName_go(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: { -uint8_t x_32; lean_object* x_33; lean_object* x_34; -lean_dec(x_22); -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_20); -return x_34; +lean_object* x_4; lean_object* x_5; uint8_t x_6; +lean_inc(x_3); +lean_inc(x_2); +x_4 = lean_name_append_index_after(x_2, x_3); +lean_inc(x_1); +lean_inc(x_4); +x_5 = lean_apply_1(x_1, x_4); +x_6 = lean_unbox(x_5); +lean_dec(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; +lean_dec(x_4); +x_7 = lean_unsigned_to_nat(1u); +x_8 = lean_nat_add(x_3, x_7); +lean_dec(x_3); +x_3 = x_8; +goto _start; } +else +{ +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_4; } } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_toVisibility___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkToParentName___closed__1() { _start: { -lean_object* x_5; -x_5 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_toVisibility(x_1, x_2, x_3, x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_5; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("to", 2, 2); +return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reduceProjs___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___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkToParentName(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_8; lean_object* x_9; -x_8 = lean_alloc_closure((void*)(l_Lean_NameSet_contains___boxed), 2, 1); -lean_closure_set(x_8, 0, x_1); +lean_object* x_3; 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; +x_3 = lean_erase_macro_scopes(x_1); +x_4 = l_Lean_Name_getString_x21(x_3); +lean_dec(x_3); +x_5 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkToParentName___closed__1; +x_6 = lean_string_append(x_5, x_4); +lean_dec(x_4); +x_7 = lean_box(0); +x_8 = l_Lean_Name_str___override(x_7, x_6); lean_inc(x_2); -x_9 = l_Lean_Meta_reduceProjOf_x3f(x_2, x_8, x_3, x_4, x_5, x_6, x_7); -if (lean_obj_tag(x_9) == 0) -{ -lean_object* x_10; -x_10 = lean_ctor_get(x_9, 0); -lean_inc(x_10); -if (lean_obj_tag(x_10) == 0) -{ -uint8_t x_11; -x_11 = !lean_is_exclusive(x_9); -if (x_11 == 0) +lean_inc(x_8); +x_9 = lean_apply_1(x_2, x_8); +x_10 = lean_unbox(x_9); +lean_dec(x_9); +if (x_10 == 0) { -lean_object* x_12; lean_object* x_13; -x_12 = lean_ctor_get(x_9, 0); -lean_dec(x_12); -x_13 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_13, 0, x_2); -lean_ctor_set(x_9, 0, x_13); -return x_9; +lean_object* x_11; lean_object* x_12; +x_11 = lean_unsigned_to_nat(1u); +x_12 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkToParentName_go(x_2, x_8, x_11); +return x_12; } else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_14 = lean_ctor_get(x_9, 1); -lean_inc(x_14); -lean_dec(x_9); -x_15 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_15, 0, x_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); -return x_16; +lean_dec(x_2); +return x_8; } } -else +} +LEAN_EXPORT uint8_t l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: { -uint8_t x_17; -lean_dec(x_2); -x_17 = !lean_is_exclusive(x_9); -if (x_17 == 0) +uint8_t x_4; +x_4 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_containsFieldName(x_1, x_3); +if (x_4 == 0) { -lean_object* x_18; uint8_t x_19; -x_18 = lean_ctor_get(x_9, 0); -lean_dec(x_18); -x_19 = !lean_is_exclusive(x_10); -if (x_19 == 0) +uint8_t x_5; +x_5 = l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(x_2, x_3); +if (x_5 == 0) { -lean_ctor_set_tag(x_10, 0); -return x_9; +uint8_t x_6; +x_6 = 1; +return x_6; } else { -lean_object* x_20; lean_object* x_21; -x_20 = lean_ctor_get(x_10, 0); -lean_inc(x_20); -lean_dec(x_10); -x_21 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_21, 0, x_20); -lean_ctor_set(x_9, 0, x_21); -return x_9; +uint8_t x_7; +x_7 = 0; +return x_7; } } else { -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_22 = lean_ctor_get(x_9, 1); -lean_inc(x_22); -lean_dec(x_9); -x_23 = lean_ctor_get(x_10, 0); -lean_inc(x_23); -if (lean_is_exclusive(x_10)) { - lean_ctor_release(x_10, 0); - x_24 = x_10; -} else { - lean_dec_ref(x_10); - x_24 = lean_box(0); -} -if (lean_is_scalar(x_24)) { - x_25 = lean_alloc_ctor(0, 1, 0); -} else { - x_25 = x_24; - lean_ctor_set_tag(x_25, 0); -} -lean_ctor_set(x_25, 0, x_23); -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_26, 1, x_22); -return x_26; -} +uint8_t x_8; +x_8 = 0; +return x_8; } } -else -{ -uint8_t x_27; -lean_dec(x_2); -x_27 = !lean_is_exclusive(x_9); -if (x_27 == 0) -{ -return x_9; } -else +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_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, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: { -lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_28 = lean_ctor_get(x_9, 0); -x_29 = lean_ctor_get(x_9, 1); -lean_inc(x_29); -lean_inc(x_28); -lean_dec(x_9); -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_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_unsigned_to_nat(1u); +x_14 = lean_nat_add(x_1, x_13); +x_15 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg(x_2, x_3, x_14, x_5, x_4, 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_Structure_0__Lean_Elab_Command_reduceProjs(lean_object* x_1, lean_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_Structure_0__Lean_Elab_Command_elabParents_go___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18) { _start: { -lean_object* x_8; lean_object* x_9; uint8_t x_10; lean_object* x_11; -x_8 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reduceProjs___lambda__1), 7, 1); -lean_closure_set(x_8, 0, x_2); -x_9 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___closed__1; -x_10 = 0; -x_11 = l_Lean_Meta_transform___at_Lean_Meta_zetaReduce___spec__1(x_1, x_9, x_8, x_10, x_10, x_3, x_4, x_5, x_6, x_7); -return x_11; +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; uint8_t x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_19 = lean_ctor_get(x_1, 4); +lean_inc(x_19); +lean_inc(x_2); +lean_inc(x_19); +x_20 = l_Lean_Name_append(x_19, x_2); +x_21 = lean_box(0); +x_22 = 3; +lean_inc(x_11); +lean_inc(x_3); +x_23 = lean_alloc_ctor(0, 5, 1); +lean_ctor_set(x_23, 0, x_3); +lean_ctor_set(x_23, 1, x_2); +lean_ctor_set(x_23, 2, x_20); +lean_ctor_set(x_23, 3, x_11); +lean_ctor_set(x_23, 4, x_21); +lean_ctor_set_uint8(x_23, sizeof(void*)*5, x_22); +x_24 = lean_array_push(x_4, x_23); +lean_inc(x_11); +x_25 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_25, 0, x_11); +x_26 = 1; +lean_inc(x_5); +x_27 = lean_alloc_ctor(0, 4, 1); +lean_ctor_set(x_27, 0, x_3); +lean_ctor_set(x_27, 1, x_25); +lean_ctor_set(x_27, 2, x_5); +lean_ctor_set(x_27, 3, x_6); +lean_ctor_set_uint8(x_27, sizeof(void*)*4, x_26); +x_28 = lean_array_push(x_7, x_27); +x_29 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg___lambda__2___boxed), 12, 4); +lean_closure_set(x_29, 0, x_8); +lean_closure_set(x_29, 1, x_1); +lean_closure_set(x_29, 2, x_9); +lean_closure_set(x_29, 3, x_28); +x_30 = lean_unsigned_to_nat(0u); +x_31 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg(x_19, x_11, x_5, x_10, x_29, x_30, x_24, x_12, x_13, x_14, x_15, x_16, x_17, x_18); +return x_31; } } -LEAN_EXPORT uint8_t l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___lambda__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { -uint8_t x_2; -x_2 = 0; -return x_2; +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; +x_17 = lean_box(0); +x_18 = 0; +lean_inc(x_3); +x_19 = lean_alloc_ctor(0, 4, 1); +lean_ctor_set(x_19, 0, x_1); +lean_ctor_set(x_19, 1, x_17); +lean_ctor_set(x_19, 2, x_2); +lean_ctor_set(x_19, 3, x_3); +lean_ctor_set_uint8(x_19, sizeof(void*)*4, x_18); +x_20 = lean_array_push(x_4, x_19); +x_21 = lean_ctor_get(x_5, 4); +lean_inc(x_21); +x_22 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg___lambda__2___boxed), 12, 4); +lean_closure_set(x_22, 0, x_6); +lean_closure_set(x_22, 1, x_5); +lean_closure_set(x_22, 2, x_7); +lean_closure_set(x_22, 3, x_20); +x_23 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom___rarg(x_21, x_8, x_3, x_22, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +return x_23; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___closed__1() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___lambda__1___boxed), 1, 0); +x_1 = l_Lean_Elab_Command_structureDiamondWarning; return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___closed__2() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___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_1; -x_1 = lean_mk_string_unchecked("ignoring default value for field '", 34, 34); -return x_1; -} +lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_13 = lean_ctor_get(x_1, 8); +lean_inc(x_13); +x_14 = lean_array_get_size(x_13); +x_15 = lean_nat_dec_lt(x_3, x_14); +lean_dec(x_14); +if (x_15 == 0) +{ +lean_object* x_16; +lean_dec(x_13); +lean_dec(x_3); +lean_dec(x_1); +x_16 = lean_apply_9(x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +return x_16; } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___closed__3() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("' defined at '", 14, 14); -return x_1; +lean_object* x_17; uint8_t x_18; +x_17 = lean_array_fget(x_13, x_3); +lean_dec(x_13); +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; +x_19 = lean_ctor_get(x_10, 2); +x_20 = lean_ctor_get(x_10, 5); +x_21 = l_Lean_replaceRef(x_17, x_20); +lean_dec(x_20); +lean_inc(x_19); +lean_ctor_set(x_10, 5, x_21); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_17); +x_22 = l_Lean_Elab_Term_elabType(x_17, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_22) == 0) +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +lean_dec(x_22); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +x_25 = lean_whnf(x_23, x_8, x_9, x_10, x_11, x_24); +if (lean_obj_tag(x_25) == 0) +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_25, 0); +lean_inc(x_26); +x_27 = lean_ctor_get(x_25, 1); +lean_inc(x_27); +lean_dec(x_25); +x_28 = l_Lean_Meta_getStructureName(x_26, 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_32; +x_29 = lean_ctor_get(x_28, 0); +lean_inc(x_29); +x_30 = lean_ctor_get(x_28, 1); +lean_inc(x_30); +lean_dec(x_28); +lean_inc(x_29); +x_31 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f(x_4, x_29, x_10, x_11, x_30); +x_32 = lean_ctor_get(x_31, 0); +lean_inc(x_32); +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; uint8_t x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; lean_object* x_43; +lean_dec(x_19); +x_33 = lean_ctor_get(x_31, 1); +lean_inc(x_33); +lean_dec(x_31); +x_34 = lean_st_ref_get(x_11, x_33); +x_35 = lean_ctor_get(x_34, 0); +lean_inc(x_35); +x_36 = lean_ctor_get(x_34, 1); +lean_inc(x_36); +lean_dec(x_34); +x_37 = lean_ctor_get(x_35, 0); +lean_inc(x_37); +lean_dec(x_35); +x_38 = 1; +lean_inc(x_29); +x_39 = l_Lean_getStructureFieldsFlattened(x_37, x_29, x_38); +lean_inc(x_39); +lean_inc(x_4); +x_40 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg___lambda__1___boxed), 3, 2); +lean_closure_set(x_40, 0, x_4); +lean_closure_set(x_40, 1, x_39); +lean_inc(x_29); +x_41 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkToParentName(x_29, x_40); +x_42 = lean_ctor_get_uint8(x_1, sizeof(void*)*12); +lean_inc(x_26); +lean_inc(x_29); +lean_inc(x_41); +x_43 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg___lambda__3___boxed), 18, 10); +lean_closure_set(x_43, 0, x_1); +lean_closure_set(x_43, 1, x_41); +lean_closure_set(x_43, 2, x_17); +lean_closure_set(x_43, 3, x_4); +lean_closure_set(x_43, 4, x_29); +lean_closure_set(x_43, 5, x_26); +lean_closure_set(x_43, 6, x_5); +lean_closure_set(x_43, 7, x_3); +lean_closure_set(x_43, 8, x_2); +lean_closure_set(x_43, 9, x_39); +if (x_42 == 0) +{ +uint8_t x_44; uint8_t x_45; lean_object* x_46; +lean_dec(x_37); +lean_dec(x_29); +x_44 = 0; +x_45 = 0; +x_46 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__1___rarg(x_41, x_44, x_26, x_43, x_45, x_6, x_7, x_8, x_9, x_10, x_11, x_36); +return x_46; } +else +{ +uint8_t x_47; +x_47 = lean_is_class(x_37, x_29); +if (x_47 == 0) +{ +uint8_t x_48; uint8_t x_49; lean_object* x_50; +x_48 = 0; +x_49 = 0; +x_50 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__1___rarg(x_41, x_48, x_26, x_43, x_49, x_6, x_7, x_8, x_9, x_10, x_11, x_36); +return x_50; } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___closed__4() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("'", 1, 1); -return x_1; +uint8_t x_51; uint8_t x_52; lean_object* x_53; +x_51 = 3; +x_52 = 0; +x_53 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__1___rarg(x_41, x_51, x_26, x_43, x_52, x_6, x_7, x_8, x_9, x_10, x_11, x_36); +return x_53; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed(lean_object* x_1, lean_object* x_2, lean_object* x_3, 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; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; 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_10 = 1; -x_11 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___closed__1; -x_12 = l_Lean_Name_toString(x_2, x_10, x_11); -x_13 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___closed__2; -x_14 = lean_string_append(x_13, x_12); -lean_dec(x_12); -x_15 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___closed__3; -x_16 = lean_string_append(x_14, x_15); -x_17 = l_Lean_Name_toString(x_1, x_10, x_11); -x_18 = lean_string_append(x_16, x_17); -lean_dec(x_17); -x_19 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___closed__4; -x_20 = lean_string_append(x_18, x_19); -x_21 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_21, 0, x_20); -x_22 = l_Lean_MessageData_ofFormat(x_21); -x_23 = l_Lean_logWarning___at_Lean_Elab_Term_mkConst___spec__4(x_22, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -x_24 = !lean_is_exclusive(x_23); -if (x_24 == 0) +lean_object* x_54; uint8_t x_55; +x_54 = lean_ctor_get(x_31, 1); +lean_inc(x_54); +lean_dec(x_31); +x_55 = !lean_is_exclusive(x_32); +if (x_55 == 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_56; lean_object* x_57; uint8_t x_58; +x_56 = lean_ctor_get(x_32, 0); +x_57 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg___closed__1; +x_58 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_19, x_57); +lean_dec(x_19); +if (x_58 == 0) +{ +lean_object* x_59; lean_object* x_60; +lean_free_object(x_32); +lean_dec(x_56); +x_59 = lean_box(0); +x_60 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg___lambda__4(x_17, x_29, x_26, x_5, x_1, x_3, x_2, x_4, x_59, x_6, x_7, x_8, x_9, x_10, x_11, x_54); +return x_60; } 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; +uint8_t x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; +x_61 = 1; +x_62 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___closed__1; +x_63 = l_Lean_Name_toString(x_56, x_61, x_62); +x_64 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__1; +x_65 = lean_string_append(x_64, x_63); +lean_dec(x_63); +x_66 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__3; +x_67 = lean_string_append(x_65, x_66); +lean_inc(x_29); +x_68 = l_Lean_Name_toString(x_29, x_61, x_62); +x_69 = lean_string_append(x_67, x_68); +lean_dec(x_68); +x_70 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__5; +x_71 = lean_string_append(x_69, x_70); +lean_ctor_set_tag(x_32, 3); +lean_ctor_set(x_32, 0, x_71); +x_72 = l_Lean_MessageData_ofFormat(x_32); +lean_inc(x_10); +x_73 = l_Lean_logWarning___at_Lean_Elab_Term_mkConst___spec__4(x_72, x_6, x_7, x_8, x_9, x_10, x_11, x_54); +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___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg___lambda__4(x_17, x_29, x_26, x_5, x_1, x_3, x_2, x_4, x_74, x_6, x_7, x_8, x_9, x_10, x_11, x_75); +lean_dec(x_74); +return x_76; } } +else +{ +lean_object* x_77; lean_object* x_78; uint8_t x_79; +x_77 = lean_ctor_get(x_32, 0); +lean_inc(x_77); +lean_dec(x_32); +x_78 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg___closed__1; +x_79 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_19, x_78); +lean_dec(x_19); +if (x_79 == 0) +{ +lean_object* x_80; lean_object* x_81; +lean_dec(x_77); +x_80 = lean_box(0); +x_81 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg___lambda__4(x_17, x_29, x_26, x_5, x_1, x_3, x_2, x_4, x_80, x_6, x_7, x_8, x_9, x_10, x_11, x_54); +return x_81; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___lambda__1___boxed(lean_object* x_1) { -_start: +else { -uint8_t x_2; lean_object* x_3; -x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___lambda__1(x_1); -lean_dec(x_1); -x_3 = lean_box(x_2); -return x_3; +uint8_t x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; +x_82 = 1; +x_83 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___closed__1; +x_84 = l_Lean_Name_toString(x_77, x_82, x_83); +x_85 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__1; +x_86 = lean_string_append(x_85, x_84); +lean_dec(x_84); +x_87 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__3; +x_88 = lean_string_append(x_86, x_87); +lean_inc(x_29); +x_89 = l_Lean_Name_toString(x_29, x_82, x_83); +x_90 = lean_string_append(x_88, x_89); +lean_dec(x_89); +x_91 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__5; +x_92 = lean_string_append(x_90, x_91); +x_93 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_93, 0, x_92); +x_94 = l_Lean_MessageData_ofFormat(x_93); +lean_inc(x_10); +x_95 = l_Lean_logWarning___at_Lean_Elab_Term_mkConst___spec__4(x_94, x_6, x_7, x_8, x_9, x_10, x_11, x_54); +x_96 = lean_ctor_get(x_95, 0); +lean_inc(x_96); +x_97 = lean_ctor_get(x_95, 1); +lean_inc(x_97); +lean_dec(x_95); +x_98 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg___lambda__4(x_17, x_29, x_26, x_5, x_1, x_3, x_2, x_4, x_96, x_6, x_7, x_8, x_9, x_10, x_11, x_97); +lean_dec(x_96); +return x_98; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +} +} +else { -lean_object* x_10; -x_10 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +uint8_t x_99; +lean_dec(x_26); +lean_dec(x_10); +lean_dec(x_19); +lean_dec(x_17); +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); lean_dec(x_3); -return x_10; -} -} -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_go_x3f___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("id", 2, 2); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_go_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_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_go_x3f___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_go_x3f(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -if (lean_obj_tag(x_5) == 6) -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; uint8_t x_17; -x_13 = lean_ctor_get(x_5, 0); -lean_inc(x_13); -x_14 = lean_ctor_get(x_5, 1); -lean_inc(x_14); -x_15 = lean_ctor_get(x_5, 2); -lean_inc(x_15); -x_16 = lean_ctor_get_uint8(x_5, sizeof(void*)*3 + 8); -lean_dec(x_5); -x_17 = l_Lean_BinderInfo_isExplicit(x_16); -if (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_dec(x_13); -x_18 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_18, 0, x_14); -x_19 = 0; -x_20 = lean_box(0); -lean_inc(x_8); -x_21 = l___private_Lean_Meta_Basic_0__Lean_Meta_mkFreshExprMVarImpl(x_18, x_19, x_20, x_8, x_9, x_10, x_11, 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 = lean_expr_instantiate1(x_15, x_22); -lean_dec(x_22); -lean_dec(x_15); -x_5 = x_24; -x_12 = x_23; -goto _start; -} -else -{ -lean_object* x_26; -x_26 = l_Lean_RBNode_find___at_Lean_NameMap_find_x3f___spec__1___rarg(x_1, x_13); -lean_dec(x_13); -if (lean_obj_tag(x_26) == 0) -{ -lean_object* x_27; -lean_dec(x_15); -lean_dec(x_14); lean_dec(x_2); -x_27 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed(x_3, x_4, 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); -return x_27; -} -else -{ -lean_object* x_28; lean_object* x_29; -x_28 = lean_ctor_get(x_26, 0); -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_28); -x_29 = lean_infer_type(x_28, x_8, x_9, x_10, x_11, x_12); -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); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -x_32 = l_Lean_Meta_isExprDefEq(x_30, x_14, x_8, x_9, x_10, x_11, x_31); -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) +lean_dec(x_1); +x_99 = !lean_is_exclusive(x_28); +if (x_99 == 0) { -lean_object* x_35; lean_object* x_36; -lean_dec(x_28); -lean_dec(x_15); -lean_dec(x_2); -x_35 = lean_ctor_get(x_32, 1); -lean_inc(x_35); -lean_dec(x_32); -x_36 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed(x_3, x_4, x_6, x_7, x_8, x_9, x_10, x_11, x_35); -lean_dec(x_11); -lean_dec(x_9); -lean_dec(x_8); -return x_36; +return x_28; } else { -lean_object* x_37; lean_object* x_38; -x_37 = lean_ctor_get(x_32, 1); -lean_inc(x_37); -lean_dec(x_32); -x_38 = lean_expr_instantiate1(x_15, x_28); +lean_object* x_100; lean_object* x_101; lean_object* x_102; +x_100 = lean_ctor_get(x_28, 0); +x_101 = lean_ctor_get(x_28, 1); +lean_inc(x_101); +lean_inc(x_100); lean_dec(x_28); -lean_dec(x_15); -x_5 = x_38; -x_12 = x_37; -goto _start; +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_40; -lean_dec(x_28); -lean_dec(x_15); -lean_dec(x_11); +uint8_t x_103; lean_dec(x_10); +lean_dec(x_19); +lean_dec(x_17); +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); lean_dec(x_3); lean_dec(x_2); -x_40 = !lean_is_exclusive(x_32); -if (x_40 == 0) +lean_dec(x_1); +x_103 = !lean_is_exclusive(x_25); +if (x_103 == 0) { -return x_32; +return x_25; } else { -lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_ctor_get(x_32, 0); -x_42 = lean_ctor_get(x_32, 1); -lean_inc(x_42); -lean_inc(x_41); -lean_dec(x_32); -x_43 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_43, 0, x_41); -lean_ctor_set(x_43, 1, x_42); -return x_43; +lean_object* x_104; lean_object* x_105; lean_object* x_106; +x_104 = lean_ctor_get(x_25, 0); +x_105 = lean_ctor_get(x_25, 1); +lean_inc(x_105); +lean_inc(x_104); +lean_dec(x_25); +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_44; -lean_dec(x_28); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_11); +uint8_t x_107; lean_dec(x_10); +lean_dec(x_19); +lean_dec(x_17); +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); lean_dec(x_3); lean_dec(x_2); -x_44 = !lean_is_exclusive(x_29); -if (x_44 == 0) +lean_dec(x_1); +x_107 = !lean_is_exclusive(x_22); +if (x_107 == 0) { -return x_29; +return x_22; } else { -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_29, 0); -x_46 = lean_ctor_get(x_29, 1); -lean_inc(x_46); -lean_inc(x_45); -lean_dec(x_29); -x_47 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_47, 0, x_45); -lean_ctor_set(x_47, 1, x_46); -return x_47; -} -} +lean_object* x_108; lean_object* x_109; lean_object* x_110; +x_108 = lean_ctor_get(x_22, 0); +x_109 = lean_ctor_get(x_22, 1); +lean_inc(x_109); +lean_inc(x_108); +lean_dec(x_22); +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_48; lean_object* x_49; uint8_t x_50; -lean_dec(x_4); -lean_dec(x_3); -x_48 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_go_x3f___closed__2; -x_49 = lean_unsigned_to_nat(2u); -x_50 = l_Lean_Expr_isAppOfArity(x_5, x_48, x_49); -if (x_50 == 0) -{ -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; -x_51 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -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___private_Lean_Elab_Structure_0__Lean_Elab_Command_reduceProjs(x_52, x_2, x_8, x_9, x_10, x_11, x_53); -if (lean_obj_tag(x_54) == 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; lean_object* x_121; uint8_t x_122; lean_object* x_123; uint8_t x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; +x_111 = lean_ctor_get(x_10, 0); +x_112 = lean_ctor_get(x_10, 1); +x_113 = lean_ctor_get(x_10, 2); +x_114 = lean_ctor_get(x_10, 3); +x_115 = lean_ctor_get(x_10, 4); +x_116 = lean_ctor_get(x_10, 5); +x_117 = lean_ctor_get(x_10, 6); +x_118 = lean_ctor_get(x_10, 7); +x_119 = lean_ctor_get(x_10, 8); +x_120 = lean_ctor_get(x_10, 9); +x_121 = lean_ctor_get(x_10, 10); +x_122 = lean_ctor_get_uint8(x_10, sizeof(void*)*12); +x_123 = lean_ctor_get(x_10, 11); +x_124 = lean_ctor_get_uint8(x_10, sizeof(void*)*12 + 1); +lean_inc(x_123); +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_inc(x_114); +lean_inc(x_113); +lean_inc(x_112); +lean_inc(x_111); +lean_dec(x_10); +x_125 = l_Lean_replaceRef(x_17, x_116); +lean_dec(x_116); +lean_inc(x_113); +x_126 = lean_alloc_ctor(0, 12, 2); +lean_ctor_set(x_126, 0, x_111); +lean_ctor_set(x_126, 1, x_112); +lean_ctor_set(x_126, 2, x_113); +lean_ctor_set(x_126, 3, x_114); +lean_ctor_set(x_126, 4, x_115); +lean_ctor_set(x_126, 5, x_125); +lean_ctor_set(x_126, 6, x_117); +lean_ctor_set(x_126, 7, x_118); +lean_ctor_set(x_126, 8, x_119); +lean_ctor_set(x_126, 9, x_120); +lean_ctor_set(x_126, 10, x_121); +lean_ctor_set(x_126, 11, x_123); +lean_ctor_set_uint8(x_126, sizeof(void*)*12, x_122); +lean_ctor_set_uint8(x_126, sizeof(void*)*12 + 1, x_124); +lean_inc(x_11); +lean_inc(x_126); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_17); +x_127 = l_Lean_Elab_Term_elabType(x_17, x_6, x_7, x_8, x_9, x_126, x_11, x_12); +if (lean_obj_tag(x_127) == 0) { -uint8_t x_55; -x_55 = !lean_is_exclusive(x_54); -if (x_55 == 0) +lean_object* x_128; lean_object* x_129; lean_object* x_130; +x_128 = lean_ctor_get(x_127, 0); +lean_inc(x_128); +x_129 = lean_ctor_get(x_127, 1); +lean_inc(x_129); +lean_dec(x_127); +lean_inc(x_11); +lean_inc(x_126); +lean_inc(x_9); +lean_inc(x_8); +x_130 = lean_whnf(x_128, x_8, x_9, x_126, x_11, x_129); +if (lean_obj_tag(x_130) == 0) { -lean_object* x_56; lean_object* x_57; -x_56 = lean_ctor_get(x_54, 0); -x_57 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_57, 0, x_56); -lean_ctor_set(x_54, 0, x_57); -return x_54; -} -else -{ -lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; -x_58 = lean_ctor_get(x_54, 0); -x_59 = lean_ctor_get(x_54, 1); -lean_inc(x_59); -lean_inc(x_58); -lean_dec(x_54); -x_60 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_60, 0, x_58); -x_61 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_61, 0, x_60); -lean_ctor_set(x_61, 1, x_59); -return x_61; -} -} -else -{ -uint8_t x_62; -x_62 = !lean_is_exclusive(x_54); -if (x_62 == 0) +lean_object* x_131; lean_object* x_132; lean_object* x_133; +x_131 = lean_ctor_get(x_130, 0); +lean_inc(x_131); +x_132 = lean_ctor_get(x_130, 1); +lean_inc(x_132); +lean_dec(x_130); +x_133 = l_Lean_Meta_getStructureName(x_131, x_8, x_9, x_126, x_11, x_132); +if (lean_obj_tag(x_133) == 0) { -return x_54; -} -else +lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; +x_134 = lean_ctor_get(x_133, 0); +lean_inc(x_134); +x_135 = lean_ctor_get(x_133, 1); +lean_inc(x_135); +lean_dec(x_133); +lean_inc(x_134); +x_136 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f(x_4, x_134, x_126, x_11, x_135); +x_137 = lean_ctor_get(x_136, 0); +lean_inc(x_137); +if (lean_obj_tag(x_137) == 0) { -lean_object* x_63; lean_object* x_64; lean_object* x_65; -x_63 = lean_ctor_get(x_54, 0); -x_64 = lean_ctor_get(x_54, 1); -lean_inc(x_64); -lean_inc(x_63); -lean_dec(x_54); -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_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; uint8_t x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; uint8_t x_147; lean_object* x_148; +lean_dec(x_113); +x_138 = lean_ctor_get(x_136, 1); +lean_inc(x_138); +lean_dec(x_136); +x_139 = lean_st_ref_get(x_11, x_138); +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 = 1; +lean_inc(x_134); +x_144 = l_Lean_getStructureFieldsFlattened(x_142, x_134, x_143); +lean_inc(x_144); +lean_inc(x_4); +x_145 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg___lambda__1___boxed), 3, 2); +lean_closure_set(x_145, 0, x_4); +lean_closure_set(x_145, 1, x_144); +lean_inc(x_134); +x_146 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkToParentName(x_134, x_145); +x_147 = lean_ctor_get_uint8(x_1, sizeof(void*)*12); +lean_inc(x_131); +lean_inc(x_134); +lean_inc(x_146); +x_148 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg___lambda__3___boxed), 18, 10); +lean_closure_set(x_148, 0, x_1); +lean_closure_set(x_148, 1, x_146); +lean_closure_set(x_148, 2, x_17); +lean_closure_set(x_148, 3, x_4); +lean_closure_set(x_148, 4, x_134); +lean_closure_set(x_148, 5, x_131); +lean_closure_set(x_148, 6, x_5); +lean_closure_set(x_148, 7, x_3); +lean_closure_set(x_148, 8, x_2); +lean_closure_set(x_148, 9, x_144); +if (x_147 == 0) +{ +uint8_t x_149; uint8_t x_150; lean_object* x_151; +lean_dec(x_142); +lean_dec(x_134); +x_149 = 0; +x_150 = 0; +x_151 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__1___rarg(x_146, x_149, x_131, x_148, x_150, x_6, x_7, x_8, x_9, x_126, x_11, x_141); +return x_151; } else { -lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; -x_66 = l_Lean_Expr_appArg_x21(x_5); -lean_dec(x_5); -x_67 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_66, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -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 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reduceProjs(x_68, x_2, x_8, x_9, x_10, x_11, x_69); -if (lean_obj_tag(x_70) == 0) -{ -uint8_t x_71; -x_71 = !lean_is_exclusive(x_70); -if (x_71 == 0) +uint8_t x_152; +x_152 = lean_is_class(x_142, x_134); +if (x_152 == 0) { -lean_object* x_72; lean_object* x_73; -x_72 = lean_ctor_get(x_70, 0); -x_73 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_73, 0, x_72); -lean_ctor_set(x_70, 0, x_73); -return x_70; +uint8_t x_153; uint8_t x_154; lean_object* x_155; +x_153 = 0; +x_154 = 0; +x_155 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__1___rarg(x_146, x_153, x_131, x_148, x_154, x_6, x_7, x_8, x_9, x_126, x_11, x_141); +return x_155; } else { -lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_74 = lean_ctor_get(x_70, 0); -x_75 = lean_ctor_get(x_70, 1); -lean_inc(x_75); -lean_inc(x_74); -lean_dec(x_70); -x_76 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_76, 0, x_74); -x_77 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_77, 0, x_76); -lean_ctor_set(x_77, 1, x_75); -return x_77; +uint8_t x_156; uint8_t x_157; lean_object* x_158; +x_156 = 3; +x_157 = 0; +x_158 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__1___rarg(x_146, x_156, x_131, x_148, x_157, x_6, x_7, x_8, x_9, x_126, x_11, x_141); +return x_158; } } -else -{ -uint8_t x_78; -x_78 = !lean_is_exclusive(x_70); -if (x_78 == 0) -{ -return x_70; } else { -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; -} -} -} +lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; uint8_t x_163; +x_159 = lean_ctor_get(x_136, 1); +lean_inc(x_159); +lean_dec(x_136); +x_160 = lean_ctor_get(x_137, 0); +lean_inc(x_160); +if (lean_is_exclusive(x_137)) { + lean_ctor_release(x_137, 0); + x_161 = x_137; +} else { + lean_dec_ref(x_137); + x_161 = lean_box(0); +} +x_162 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg___closed__1; +x_163 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_113, x_162); +lean_dec(x_113); +if (x_163 == 0) +{ +lean_object* x_164; lean_object* x_165; +lean_dec(x_161); +lean_dec(x_160); +x_164 = lean_box(0); +x_165 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg___lambda__4(x_17, x_134, x_131, x_5, x_1, x_3, x_2, x_4, x_164, x_6, x_7, x_8, x_9, x_126, x_11, x_159); +return x_165; +} +else +{ +uint8_t 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_166 = 1; +x_167 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___closed__1; +x_168 = l_Lean_Name_toString(x_160, x_166, x_167); +x_169 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__1; +x_170 = lean_string_append(x_169, x_168); +lean_dec(x_168); +x_171 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__3; +x_172 = lean_string_append(x_170, x_171); +lean_inc(x_134); +x_173 = l_Lean_Name_toString(x_134, x_166, x_167); +x_174 = lean_string_append(x_172, x_173); +lean_dec(x_173); +x_175 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__5; +x_176 = lean_string_append(x_174, x_175); +if (lean_is_scalar(x_161)) { + x_177 = lean_alloc_ctor(3, 1, 0); +} else { + x_177 = x_161; + lean_ctor_set_tag(x_177, 3); +} +lean_ctor_set(x_177, 0, x_176); +x_178 = l_Lean_MessageData_ofFormat(x_177); +lean_inc(x_126); +x_179 = l_Lean_logWarning___at_Lean_Elab_Term_mkConst___spec__4(x_178, x_6, x_7, x_8, x_9, x_126, x_11, x_159); +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___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg___lambda__4(x_17, x_134, x_131, x_5, x_1, x_3, x_2, x_4, x_180, x_6, x_7, x_8, x_9, x_126, x_11, x_181); +lean_dec(x_180); +return x_182; } } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_go_x3f___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: +else { -lean_object* x_13; -x_13 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_go_x3f(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_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; +lean_dec(x_131); +lean_dec(x_126); +lean_dec(x_113); +lean_dec(x_17); +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); +lean_dec(x_3); +lean_dec(x_2); lean_dec(x_1); -return x_13; +x_183 = lean_ctor_get(x_133, 0); +lean_inc(x_183); +x_184 = lean_ctor_get(x_133, 1); +lean_inc(x_184); +if (lean_is_exclusive(x_133)) { + lean_ctor_release(x_133, 0); + lean_ctor_release(x_133, 1); + x_185 = x_133; +} else { + lean_dec_ref(x_133); + x_185 = lean_box(0); } +if (lean_is_scalar(x_185)) { + x_186 = lean_alloc_ctor(1, 2, 0); +} else { + x_186 = x_185; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -lean_object* x_12; uint8_t x_13; -x_12 = lean_st_ref_get(x_10, x_11); -x_13 = !lean_is_exclusive(x_12); -if (x_13 == 0) -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; -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); -lean_inc(x_4); -lean_inc(x_3); -x_17 = l_Lean_getDefaultFnForField_x3f(x_16, x_3, x_4); -if (lean_obj_tag(x_17) == 0) +lean_ctor_set(x_186, 0, x_183); +lean_ctor_set(x_186, 1, x_184); +return x_186; +} +} +else { -lean_object* x_18; -lean_dec(x_10); +lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; +lean_dec(x_126); +lean_dec(x_113); +lean_dec(x_17); +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); lean_dec(x_3); lean_dec(x_2); -x_18 = lean_box(0); -lean_ctor_set(x_12, 0, x_18); -return x_12; +lean_dec(x_1); +x_187 = lean_ctor_get(x_130, 0); +lean_inc(x_187); +x_188 = lean_ctor_get(x_130, 1); +lean_inc(x_188); +if (lean_is_exclusive(x_130)) { + lean_ctor_release(x_130, 0); + lean_ctor_release(x_130, 1); + x_189 = x_130; +} else { + lean_dec_ref(x_130); + x_189 = lean_box(0); +} +if (lean_is_scalar(x_189)) { + x_190 = lean_alloc_ctor(1, 2, 0); +} else { + x_190 = x_189; +} +lean_ctor_set(x_190, 0, x_187); +lean_ctor_set(x_190, 1, x_188); +return x_190; } -else -{ -lean_object* x_19; lean_object* x_20; -lean_free_object(x_12); -x_19 = lean_ctor_get(x_17, 0); -lean_inc(x_19); -lean_dec(x_17); -lean_inc(x_5); -x_20 = l_Lean_getConstInfo___at_Lean_Elab_Term_mkConst___spec__1(x_19, x_5, x_6, x_7, x_8, x_9, x_10, x_15); -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; -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_Meta_mkFreshLevelMVarsFor(x_21, x_7, x_8, x_9, x_10, x_22); -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_23, 1); -lean_inc(x_25); -lean_dec(x_23); -x_26 = l_Lean_Core_instantiateValueLevelParams(x_21, x_24, x_9, x_10, x_25); -lean_dec(x_21); -if (lean_obj_tag(x_26) == 0) -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_26, 0); -lean_inc(x_27); -x_28 = lean_ctor_get(x_26, 1); -lean_inc(x_28); -lean_dec(x_26); -x_29 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_go_x3f(x_1, x_2, x_3, x_4, x_27, x_5, x_6, x_7, x_8, x_9, x_10, x_28); -lean_dec(x_5); -return x_29; } else { -uint8_t x_30; -lean_dec(x_10); +lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; +lean_dec(x_126); +lean_dec(x_113); +lean_dec(x_17); +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); lean_dec(x_3); lean_dec(x_2); -x_30 = !lean_is_exclusive(x_26); -if (x_30 == 0) -{ -return x_26; +lean_dec(x_1); +x_191 = lean_ctor_get(x_127, 0); +lean_inc(x_191); +x_192 = lean_ctor_get(x_127, 1); +lean_inc(x_192); +if (lean_is_exclusive(x_127)) { + lean_ctor_release(x_127, 0); + lean_ctor_release(x_127, 1); + x_193 = x_127; +} else { + lean_dec_ref(x_127); + x_193 = lean_box(0); } -else -{ -lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_31 = lean_ctor_get(x_26, 0); -x_32 = lean_ctor_get(x_26, 1); -lean_inc(x_32); -lean_inc(x_31); -lean_dec(x_26); -x_33 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_33, 0, x_31); -lean_ctor_set(x_33, 1, x_32); -return x_33; +if (lean_is_scalar(x_193)) { + x_194 = lean_alloc_ctor(1, 2, 0); +} else { + x_194 = x_193; } +lean_ctor_set(x_194, 0, x_191); +lean_ctor_set(x_194, 1, x_192); +return x_194; } } -else -{ -uint8_t x_34; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_34 = !lean_is_exclusive(x_20); -if (x_34 == 0) -{ -return x_20; } -else -{ -lean_object* x_35; lean_object* x_36; lean_object* x_37; -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_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_Elab_Structure_0__Lean_Elab_Command_elabParents_go(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg), 12, 0); +return x_2; } } -else -{ -lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_38 = lean_ctor_get(x_12, 0); -x_39 = lean_ctor_get(x_12, 1); -lean_inc(x_39); -lean_inc(x_38); -lean_dec(x_12); -x_40 = lean_ctor_get(x_38, 0); -lean_inc(x_40); -lean_dec(x_38); -lean_inc(x_4); -lean_inc(x_3); -x_41 = l_Lean_getDefaultFnForField_x3f(x_40, x_3, x_4); -if (lean_obj_tag(x_41) == 0) +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: { -lean_object* x_42; lean_object* x_43; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_5); -lean_dec(x_4); +uint8_t x_4; lean_object* x_5; +x_4 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg___lambda__1(x_1, x_2, x_3); lean_dec(x_3); lean_dec(x_2); -x_42 = lean_box(0); -x_43 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_43, 0, x_42); -lean_ctor_set(x_43, 1, x_39); -return x_43; +lean_dec(x_1); +x_5 = lean_box(x_4); +return x_5; } -else -{ -lean_object* x_44; lean_object* x_45; -x_44 = lean_ctor_get(x_41, 0); -lean_inc(x_44); -lean_dec(x_41); -lean_inc(x_5); -x_45 = l_Lean_getConstInfo___at_Lean_Elab_Term_mkConst___spec__1(x_44, x_5, x_6, x_7, x_8, x_9, x_10, x_39); -if (lean_obj_tag(x_45) == 0) -{ -lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_46 = lean_ctor_get(x_45, 0); -lean_inc(x_46); -x_47 = lean_ctor_get(x_45, 1); -lean_inc(x_47); -lean_dec(x_45); -x_48 = l_Lean_Meta_mkFreshLevelMVarsFor(x_46, x_7, x_8, x_9, x_10, 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 = l_Lean_Core_instantiateValueLevelParams(x_46, x_49, x_9, x_10, x_50); -lean_dec(x_46); -if (lean_obj_tag(x_51) == 0) -{ -lean_object* x_52; lean_object* x_53; lean_object* 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___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_go_x3f(x_1, x_2, x_3, x_4, x_52, x_5, x_6, x_7, x_8, x_9, x_10, x_53); -lean_dec(x_5); -return x_54; } -else +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_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, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: { -lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_55 = lean_ctor_get(x_51, 0); -lean_inc(x_55); -x_56 = lean_ctor_get(x_51, 1); -lean_inc(x_56); -if (lean_is_exclusive(x_51)) { - lean_ctor_release(x_51, 0); - lean_ctor_release(x_51, 1); - x_57 = x_51; -} else { - lean_dec_ref(x_51); - x_57 = lean_box(0); +lean_object* x_13; +x_13 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_1); +return x_13; } -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_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___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]; +lean_object* x_18 = _args[17]; +_start: +{ +lean_object* x_19; +x_19 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18); +return x_19; } } -else +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +_start: { -lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; -lean_dec(x_10); +lean_object* x_17; +x_17 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_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; -} else { - lean_dec_ref(x_45); - x_61 = lean_box(0); +return x_17; } -if (lean_is_scalar(x_61)) { - x_62 = lean_alloc_ctor(1, 2, 0); -} else { - x_62 = x_61; } -lean_ctor_set(x_62, 0, x_59); -lean_ctor_set(x_62, 1, x_60); -return x_62; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents___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; +x_10 = lean_unsigned_to_nat(0u); +x_11 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__1; +x_12 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg(x_1, x_2, x_10, x_11, x_11, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_12; +} } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents___rarg), 9, 0); +return x_2; } } +LEAN_EXPORT uint8_t l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabFieldTypeValue___lambda__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; uint8_t x_4; +x_3 = lean_ctor_get(x_1, 4); +x_4 = lean_name_eq(x_3, x_2); +return x_4; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabFieldTypeValue___lambda__2___closed__1() { _start: { -lean_object* x_12; -x_12 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_6); -lean_dec(x_1); -return x_12; +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +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_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_processOveriddenDefaultValues___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabFieldTypeValue___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -uint8_t x_14; -x_14 = lean_usize_dec_lt(x_5, x_4); -if (x_14 == 0) +lean_object* x_10; +x_10 = lean_ctor_get(x_1, 7); +lean_inc(x_10); +if (lean_obj_tag(x_10) == 0) { -lean_object* x_15; -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); +lean_object* x_11; +x_11 = lean_ctor_get(x_1, 8); +lean_inc(x_11); +lean_dec(x_1); +if (lean_obj_tag(x_11) == 0) +{ +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_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_12 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabFieldTypeValue___lambda__2___closed__1; +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_9); +return x_13; } 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; lean_object* x_23; -x_16 = lean_array_uget(x_6, x_5); -x_17 = lean_unsigned_to_nat(0u); -x_18 = lean_array_uset(x_6, x_5, x_17); -x_19 = lean_ctor_get(x_16, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_16, 1); -lean_inc(x_20); -x_21 = lean_ctor_get(x_16, 2); -lean_inc(x_21); -x_22 = lean_ctor_get_uint8(x_16, sizeof(void*)*4); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); +uint8_t x_14; +x_14 = !lean_is_exclusive(x_11); +if (x_14 == 0) +{ +lean_object* x_15; uint8_t x_16; uint8_t x_17; lean_object* x_18; +x_15 = lean_ctor_get(x_11, 0); +x_16 = 1; +x_17 = 0; +lean_inc(x_8); lean_inc(x_7); -lean_inc(x_19); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); lean_inc(x_3); -lean_inc(x_2); -x_23 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f(x_1, x_2, x_3, x_19, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_23) == 0) +x_18 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_16, x_17, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_18) == 0) { -lean_object* x_24; -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -if (lean_obj_tag(x_24) == 0) +lean_object* x_19; lean_object* x_20; +x_19 = lean_ctor_get(x_18, 1); +lean_inc(x_19); +lean_dec(x_18); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_3); +x_20 = l_Lean_Elab_Term_addAutoBoundImplicits(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_19); +if (lean_obj_tag(x_20) == 0) { -lean_object* x_25; size_t x_26; size_t x_27; lean_object* x_28; -lean_dec(x_21); +lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +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_dec(x_19); -x_25 = lean_ctor_get(x_23, 1); -lean_inc(x_25); -lean_dec(x_23); -x_26 = 1; -x_27 = lean_usize_add(x_5, x_26); -x_28 = lean_array_uset(x_18, x_5, x_16); -x_5 = x_27; -x_6 = x_28; -x_13 = x_25; -goto _start; -} -else +x_23 = lean_box(0); +x_24 = 1; +x_25 = lean_box(x_24); +x_26 = lean_box(x_24); +x_27 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTerm___boxed), 11, 4); +lean_closure_set(x_27, 0, x_15); +lean_closure_set(x_27, 1, x_23); +lean_closure_set(x_27, 2, x_25); +lean_closure_set(x_27, 3, x_26); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_28 = l_Lean_Elab_Term_withoutAutoBoundImplicit___rarg(x_27, x_3, x_4, x_5, x_6, x_7, x_8, x_22); +if (lean_obj_tag(x_28) == 0) { -uint8_t x_30; -x_30 = !lean_is_exclusive(x_16); -if (x_30 == 0) +lean_object* x_29; lean_object* x_30; uint8_t x_31; lean_object* x_32; +x_29 = lean_ctor_get(x_28, 0); +lean_inc(x_29); +x_30 = lean_ctor_get(x_28, 1); +lean_inc(x_30); +lean_dec(x_28); +x_31 = 1; +x_32 = l_Lean_Meta_mkLambdaFVars(x_21, x_29, x_17, x_24, x_17, x_31, 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); +if (lean_obj_tag(x_32) == 0) { -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; -x_31 = lean_ctor_get(x_16, 3); -lean_dec(x_31); -x_32 = lean_ctor_get(x_16, 2); -lean_dec(x_32); -x_33 = lean_ctor_get(x_16, 1); -lean_dec(x_33); -x_34 = lean_ctor_get(x_16, 0); -lean_dec(x_34); -x_35 = lean_ctor_get(x_23, 1); -lean_inc(x_35); -lean_dec(x_23); -x_36 = !lean_is_exclusive(x_24); -if (x_36 == 0) +uint8_t x_33; +x_33 = !lean_is_exclusive(x_32); +if (x_33 == 0) { -size_t x_37; size_t x_38; lean_object* x_39; -lean_ctor_set(x_16, 3, x_24); -x_37 = 1; -x_38 = lean_usize_add(x_5, x_37); -x_39 = lean_array_uset(x_18, x_5, x_16); -x_5 = x_38; -x_6 = x_39; -x_13 = x_35; -goto _start; +lean_object* x_34; lean_object* x_35; +x_34 = lean_ctor_get(x_32, 0); +lean_ctor_set(x_11, 0, x_34); +x_35 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_35, 0, x_23); +lean_ctor_set(x_35, 1, x_11); +lean_ctor_set(x_32, 0, x_35); +return x_32; } else { -lean_object* x_41; lean_object* x_42; size_t x_43; size_t x_44; lean_object* x_45; -x_41 = lean_ctor_get(x_24, 0); -lean_inc(x_41); -lean_dec(x_24); -x_42 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_42, 0, x_41); -lean_ctor_set(x_16, 3, x_42); -x_43 = 1; -x_44 = lean_usize_add(x_5, x_43); -x_45 = lean_array_uset(x_18, x_5, x_16); -x_5 = x_44; -x_6 = x_45; -x_13 = x_35; -goto _start; +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); +lean_ctor_set(x_11, 0, x_36); +x_38 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_38, 0, x_23); +lean_ctor_set(x_38, 1, x_11); +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_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; size_t x_52; size_t x_53; lean_object* x_54; -lean_dec(x_16); -x_47 = lean_ctor_get(x_23, 1); -lean_inc(x_47); -lean_dec(x_23); -x_48 = lean_ctor_get(x_24, 0); -lean_inc(x_48); -if (lean_is_exclusive(x_24)) { - lean_ctor_release(x_24, 0); - x_49 = x_24; -} else { - lean_dec_ref(x_24); - x_49 = lean_box(0); -} -if (lean_is_scalar(x_49)) { - x_50 = lean_alloc_ctor(1, 1, 0); -} else { - x_50 = x_49; +uint8_t x_40; +lean_free_object(x_11); +x_40 = !lean_is_exclusive(x_32); +if (x_40 == 0) +{ +return x_32; } -lean_ctor_set(x_50, 0, x_48); -x_51 = lean_alloc_ctor(0, 4, 1); -lean_ctor_set(x_51, 0, x_19); -lean_ctor_set(x_51, 1, x_20); -lean_ctor_set(x_51, 2, x_21); -lean_ctor_set(x_51, 3, x_50); -lean_ctor_set_uint8(x_51, sizeof(void*)*4, x_22); -x_52 = 1; -x_53 = lean_usize_add(x_5, x_52); -x_54 = lean_array_uset(x_18, x_5, x_51); -x_5 = x_53; -x_6 = x_54; -x_13 = x_47; -goto _start; +else +{ +lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_41 = lean_ctor_get(x_32, 0); +x_42 = lean_ctor_get(x_32, 1); +lean_inc(x_42); +lean_inc(x_41); +lean_dec(x_32); +x_43 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_43, 0, x_41); +lean_ctor_set(x_43, 1, x_42); +return x_43; } } } else { -uint8_t x_56; +uint8_t x_44; lean_dec(x_21); -lean_dec(x_20); -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_16); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); +lean_free_object(x_11); +lean_dec(x_8); lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -x_56 = !lean_is_exclusive(x_23); -if (x_56 == 0) +lean_dec(x_6); +lean_dec(x_5); +x_44 = !lean_is_exclusive(x_28); +if (x_44 == 0) { -return x_23; +return x_28; } else { -lean_object* x_57; lean_object* x_58; lean_object* x_59; -x_57 = lean_ctor_get(x_23, 0); -x_58 = lean_ctor_get(x_23, 1); -lean_inc(x_58); -lean_inc(x_57); -lean_dec(x_23); -x_59 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_59, 0, x_57); -lean_ctor_set(x_59, 1, x_58); -return x_59; -} -} -} -} +lean_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_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_processOveriddenDefaultValues(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, 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_array_size(x_1); -x_13 = 0; -x_14 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_processOveriddenDefaultValues___spec__1(x_2, x_3, x_4, x_12, x_13, x_1, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -return x_14; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_processOveriddenDefaultValues___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { -_start: +else { -size_t x_14; size_t x_15; lean_object* x_16; -x_14 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_15 = lean_unbox_usize(x_5); -lean_dec(x_5); -x_16 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_processOveriddenDefaultValues___spec__1(x_1, x_2, x_3, x_14, x_15, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +uint8_t x_48; +lean_free_object(x_11); +lean_dec(x_15); lean_dec(x_8); -lean_dec(x_1); -return x_16; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_processOveriddenDefaultValues___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -lean_object* x_12; -x_12 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_processOveriddenDefaultValues(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_7); lean_dec(x_6); -lean_dec(x_2); -return x_12; -} -} -static lean_object* _init_l_panic___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___spec__1___closed__1() { -_start: +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_48 = !lean_is_exclusive(x_20); +if (x_48 == 0) { -lean_object* x_1; -x_1 = l_Lean_Elab_Term_instInhabitedTermElabM(lean_box(0)); -return x_1; -} +return x_20; } -LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___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: +else { -lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_9 = l_panic___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___spec__1___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_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; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___spec__2___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("failed to copy fields from parent structure", 43, 43); -return x_1; } +else +{ +uint8_t x_52; +lean_free_object(x_11); +lean_dec(x_15); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_52 = !lean_is_exclusive(x_18); +if (x_52 == 0) +{ +return x_18; } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___spec__2___closed__2() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___spec__2___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +lean_object* x_53; lean_object* x_54; lean_object* x_55; +x_53 = lean_ctor_get(x_18, 0); +x_54 = lean_ctor_get(x_18, 1); +lean_inc(x_54); +lean_inc(x_53); +lean_dec(x_18); +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_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___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: -{ -uint8_t x_14; -x_14 = lean_usize_dec_lt(x_5, x_4); -if (x_14 == 0) -{ -lean_object* x_15; -lean_dec(x_7); -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_16; lean_object* x_17; -x_16 = lean_array_uget(x_3, x_5); -x_17 = l_Lean_RBNode_find___at_Lean_NameMap_find_x3f___spec__1___rarg(x_2, x_16); -lean_dec(x_16); -if (lean_obj_tag(x_17) == 0) +lean_object* x_56; uint8_t x_57; uint8_t x_58; lean_object* x_59; +x_56 = lean_ctor_get(x_11, 0); +lean_inc(x_56); +lean_dec(x_11); +x_57 = 1; +x_58 = 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_59 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_57, x_58, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_59) == 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_60; lean_object* x_61; +x_60 = lean_ctor_get(x_59, 1); +lean_inc(x_60); +lean_dec(x_59); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_3); +x_61 = l_Lean_Elab_Term_addAutoBoundImplicits(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_60); +if (lean_obj_tag(x_61) == 0) +{ +lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; +x_62 = lean_ctor_get(x_61, 0); +lean_inc(x_62); +x_63 = lean_ctor_get(x_61, 1); +lean_inc(x_63); +lean_dec(x_61); +x_64 = lean_box(0); +x_65 = 1; +x_66 = lean_box(x_65); +x_67 = lean_box(x_65); +x_68 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTerm___boxed), 11, 4); +lean_closure_set(x_68, 0, x_56); +lean_closure_set(x_68, 1, x_64); +lean_closure_set(x_68, 2, x_66); +lean_closure_set(x_68, 3, x_67); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_69 = l_Lean_Elab_Term_withoutAutoBoundImplicit___rarg(x_68, x_3, x_4, x_5, x_6, x_7, x_8, x_63); +if (lean_obj_tag(x_69) == 0) +{ +lean_object* x_70; lean_object* x_71; uint8_t x_72; lean_object* x_73; +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 = 1; +x_73 = l_Lean_Meta_mkLambdaFVars(x_62, x_70, x_58, x_65, x_58, x_72, x_5, x_6, x_7, x_8, x_71); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); -x_18 = l_Lean_indentExpr(x_1); -x_19 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___spec__2___closed__2; -x_20 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_20, 0, x_19); -lean_ctor_set(x_20, 1, x_18); -x_21 = l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__4; -x_22 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_22, 0, x_20); -lean_ctor_set(x_22, 1, x_21); -x_23 = l_Lean_throwError___at_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) +lean_dec(x_5); +if (lean_obj_tag(x_73) == 0) { -return x_23; +lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; +x_74 = lean_ctor_get(x_73, 0); +lean_inc(x_74); +x_75 = lean_ctor_get(x_73, 1); +lean_inc(x_75); +if (lean_is_exclusive(x_73)) { + lean_ctor_release(x_73, 0); + lean_ctor_release(x_73, 1); + x_76 = x_73; +} else { + lean_dec_ref(x_73); + x_76 = lean_box(0); } -else -{ -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_23, 0); -x_26 = lean_ctor_get(x_23, 1); -lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_23); -x_27 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_26); -return x_27; +x_77 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_77, 0, x_74); +x_78 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_78, 0, x_64); +lean_ctor_set(x_78, 1, x_77); +if (lean_is_scalar(x_76)) { + x_79 = lean_alloc_ctor(0, 2, 0); +} else { + x_79 = x_76; } +lean_ctor_set(x_79, 0, x_78); +lean_ctor_set(x_79, 1, x_75); +return x_79; } else { -lean_object* x_28; lean_object* x_29; size_t x_30; size_t x_31; -x_28 = lean_ctor_get(x_17, 0); -lean_inc(x_28); -lean_dec(x_17); -x_29 = l_Lean_Expr_app___override(x_6, x_28); -x_30 = 1; -x_31 = lean_usize_add(x_5, x_30); -x_5 = x_31; -x_6 = x_29; -goto _start; -} -} +lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; +x_80 = lean_ctor_get(x_73, 0); +lean_inc(x_80); +x_81 = lean_ctor_get(x_73, 1); +lean_inc(x_81); +if (lean_is_exclusive(x_73)) { + lean_ctor_release(x_73, 0); + lean_ctor_release(x_73, 1); + x_82 = x_73; +} else { + lean_dec_ref(x_73); + x_82 = lean_box(0); } +if (lean_is_scalar(x_82)) { + x_83 = lean_alloc_ctor(1, 2, 0); +} else { + x_83 = x_82; } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Lean.Elab.Structure", 19, 19); -return x_1; +lean_ctor_set(x_83, 0, x_80); +lean_ctor_set(x_83, 1, x_81); +return x_83; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__2() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("_private.Lean.Elab.Structure.0.Lean.Elab.Command.copyNewFieldsFrom.mkCompositeField", 83, 83); -return x_1; +lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; +lean_dec(x_62); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_84 = lean_ctor_get(x_69, 0); +lean_inc(x_84); +x_85 = lean_ctor_get(x_69, 1); +lean_inc(x_85); +if (lean_is_exclusive(x_69)) { + lean_ctor_release(x_69, 0); + lean_ctor_release(x_69, 1); + x_86 = x_69; +} else { + lean_dec_ref(x_69); + x_86 = lean_box(0); } +if (lean_is_scalar(x_86)) { + x_87 = lean_alloc_ctor(1, 2, 0); +} else { + x_87 = x_86; } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("unreachable code has been reached", 33, 33); -return x_1; +lean_ctor_set(x_87, 0, x_84); +lean_ctor_set(x_87, 1, x_85); +return x_87; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___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___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__1; -x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__2; -x_3 = lean_unsigned_to_nat(450u); -x_4 = lean_unsigned_to_nat(68u); -x_5 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__3; -x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); -return x_6; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField(lean_object* x_1, lean_object* x_2, lean_object* x_3, 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 = lean_st_ref_get(x_8, x_9); -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -x_12 = lean_ctor_get(x_10, 1); -lean_inc(x_12); -lean_dec(x_10); -x_13 = lean_ctor_get(x_11, 0); -lean_inc(x_13); -lean_dec(x_11); -x_14 = l_Lean_Expr_getAppFn(x_1); -if (lean_obj_tag(x_14) == 4) -{ -lean_object* x_15; lean_object* x_16; 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; size_t x_30; size_t x_31; lean_object* x_32; -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_15); -lean_inc(x_13); -x_17 = l_Lean_getStructureCtor(x_13, x_15); -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 = l_Lean_Expr_const___override(x_19, x_16); -x_21 = lean_unsigned_to_nat(0u); -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); -x_25 = lean_unsigned_to_nat(1u); -x_26 = lean_nat_sub(x_22, x_25); -lean_dec(x_22); -lean_inc(x_1); -x_27 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_1, x_24, x_26); -x_28 = l_Lean_mkAppN(x_20, x_27); -lean_dec(x_27); -x_29 = l_Lean_getStructureFields(x_13, x_15); -lean_dec(x_13); -x_30 = lean_array_size(x_29); -x_31 = 0; -x_32 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___spec__2(x_1, x_2, x_29, x_30, x_31, x_28, x_3, x_4, x_5, x_6, x_7, x_8, x_12); +lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; +lean_dec(x_56); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_29); -if (lean_obj_tag(x_32) == 0) -{ -uint8_t x_33; -x_33 = !lean_is_exclusive(x_32); -if (x_33 == 0) -{ -return x_32; -} -else -{ -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_32, 0); -x_35 = lean_ctor_get(x_32, 1); -lean_inc(x_35); -lean_inc(x_34); -lean_dec(x_32); -x_36 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_36, 0, x_34); -lean_ctor_set(x_36, 1, x_35); -return x_36; -} -} -else -{ -uint8_t x_37; -x_37 = !lean_is_exclusive(x_32); -if (x_37 == 0) -{ -return x_32; -} -else -{ -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_32, 0); -x_39 = lean_ctor_get(x_32, 1); -lean_inc(x_39); -lean_inc(x_38); -lean_dec(x_32); -x_40 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_40, 0, x_38); -lean_ctor_set(x_40, 1, x_39); -return x_40; -} -} -} -else -{ -lean_object* x_41; lean_object* x_42; -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_1); -x_41 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__4; -x_42 = l_panic___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___spec__1(x_41, x_3, x_4, x_5, x_6, x_7, x_8, x_12); -return x_42; -} -} -} -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { -_start: -{ -size_t x_14; size_t x_15; lean_object* x_16; -x_14 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_15 = lean_unbox_usize(x_5); -lean_dec(x_5); -x_16 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___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_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); lean_dec(x_3); -lean_dec(x_2); -return x_16; -} +x_88 = lean_ctor_get(x_61, 0); +lean_inc(x_88); +x_89 = lean_ctor_get(x_61, 1); +lean_inc(x_89); +if (lean_is_exclusive(x_61)) { + lean_ctor_release(x_61, 0); + lean_ctor_release(x_61, 1); + x_90 = x_61; +} else { + lean_dec_ref(x_61); + x_90 = lean_box(0); } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; -x_10 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField(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; +if (lean_is_scalar(x_90)) { + x_91 = lean_alloc_ctor(1, 2, 0); +} else { + x_91 = x_90; } +lean_ctor_set(x_91, 0, x_88); +lean_ctor_set(x_91, 1, x_89); +return x_91; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields___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_13; -x_13 = l_Lean_Meta_getStructureName(x_4, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_13) == 0) -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_14 = lean_ctor_get(x_13, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_13, 1); -lean_inc(x_15); -lean_dec(x_13); -x_16 = lean_st_ref_get(x_11, x_15); -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_16, 1); -lean_inc(x_18); -lean_dec(x_16); -x_19 = lean_ctor_get(x_17, 0); -lean_inc(x_19); -lean_dec(x_17); -lean_inc(x_14); -x_20 = l_Lean_getStructureFields(x_19, x_14); -lean_dec(x_19); -x_21 = lean_box(0); -x_22 = lean_unsigned_to_nat(0u); -x_23 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg(x_1, x_4, x_5, x_14, x_20, x_22, x_2, x_21, x_3, x_6, x_7, x_8, x_9, x_10, x_11, x_18); -return x_23; } else { -uint8_t x_24; -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); +lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; +lean_dec(x_56); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_24 = !lean_is_exclusive(x_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; +x_92 = lean_ctor_get(x_59, 0); +lean_inc(x_92); +x_93 = lean_ctor_get(x_59, 1); +lean_inc(x_93); +if (lean_is_exclusive(x_59)) { + lean_ctor_release(x_59, 0); + lean_ctor_release(x_59, 1); + x_94 = x_59; +} else { + lean_dec_ref(x_59); + x_94 = lean_box(0); } +if (lean_is_scalar(x_94)) { + x_95 = lean_alloc_ctor(1, 2, 0); +} else { + x_95 = x_94; } +lean_ctor_set(x_95, 0, x_92); +lean_ctor_set(x_95, 1, x_93); +return x_95; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields___rarg), 12, 0); -return x_2; } } -LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___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: +else { -lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_9 = l_panic___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___spec__1___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_EXPORT lean_object* l_panic___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___spec__1(lean_object* x_1) { -_start: +uint8_t x_96; +x_96 = !lean_is_exclusive(x_10); +if (x_96 == 0) { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_panic___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___spec__1___rarg), 8, 0); -return x_2; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19, lean_object* x_20) { -_start: -{ -lean_object* x_21; lean_object* x_22; -lean_inc(x_13); -lean_inc(x_2); -x_21 = l_Lean_RBNode_insert___at_Lean_NameMap_insert___spec__1___rarg(x_1, x_2, x_13); -lean_inc(x_19); -lean_inc(x_18); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_14); -lean_inc(x_2); +lean_object* x_97; lean_object* x_98; +x_97 = 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_22 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f(x_21, x_3, x_4, x_2, x_14, x_15, x_16, x_17, x_18, x_19, x_20); -if (lean_obj_tag(x_22) == 0) +x_98 = l_Lean_Elab_Term_elabType(x_97, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_98) == 0) { -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; lean_object* x_30; -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -x_24 = lean_ctor_get(x_22, 1); -lean_inc(x_24); -lean_dec(x_22); -lean_inc(x_2); +lean_object* x_99; lean_object* x_100; uint8_t x_101; uint8_t x_102; lean_object* x_103; +x_99 = lean_ctor_get(x_98, 0); +lean_inc(x_99); +x_100 = lean_ctor_get(x_98, 1); +lean_inc(x_100); +lean_dec(x_98); +x_101 = 1; +x_102 = 0; +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); lean_inc(x_5); -x_25 = l_Lean_Name_append(x_5, x_2); -x_26 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_toVisibility(x_6, x_18, x_19, x_24); -x_27 = lean_ctor_get(x_26, 0); -lean_inc(x_27); -x_28 = lean_ctor_get(x_26, 1); -lean_inc(x_28); -lean_dec(x_26); -x_29 = lean_unbox(x_27); -lean_dec(x_27); -lean_inc(x_14); -x_30 = l_Lean_Elab_applyVisibility___at_Lean_Elab_Term_expandDeclId___spec__5(x_29, x_25, x_14, x_15, x_16, x_17, x_18, x_19, x_28); -if (lean_obj_tag(x_30) == 0) +lean_inc(x_4); +lean_inc(x_3); +x_103 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_101, x_102, x_3, x_4, x_5, x_6, x_7, x_8, x_100); +if (lean_obj_tag(x_103) == 0) { -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; -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_st_ref_get(x_19, x_32); -x_34 = lean_ctor_get(x_33, 0); -lean_inc(x_34); -x_35 = lean_ctor_get(x_33, 1); -lean_inc(x_35); -lean_dec(x_33); -x_36 = lean_ctor_get(x_34, 0); -lean_inc(x_36); -lean_dec(x_34); -x_37 = 1; -x_38 = l_Lean_findDocString_x3f(x_36, x_7, x_37, x_35); -lean_dec(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); -lean_inc(x_14); -lean_inc(x_31); -x_41 = l_Lean_addDocString_x27___at_Lean_Elab_Term_expandDeclId___spec__8(x_31, x_39, x_14, x_15, x_16, x_17, x_18, x_19, x_40); -if (lean_obj_tag(x_41) == 0) +lean_object* x_104; lean_object* x_105; +x_104 = lean_ctor_get(x_103, 1); +lean_inc(x_104); +lean_dec(x_103); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_3); +x_105 = l_Lean_Elab_Term_addAutoBoundImplicits(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_104); +if (lean_obj_tag(x_105) == 0) { -lean_object* x_42; uint8_t x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; -x_42 = lean_ctor_get(x_41, 1); -lean_inc(x_42); -lean_dec(x_41); -x_43 = 1; -x_44 = lean_alloc_ctor(0, 4, 1); -lean_ctor_set(x_44, 0, x_2); -lean_ctor_set(x_44, 1, x_31); -lean_ctor_set(x_44, 2, x_13); -lean_ctor_set(x_44, 3, x_23); -lean_ctor_set_uint8(x_44, sizeof(void*)*4, x_43); -x_45 = lean_array_push(x_8, x_44); -x_46 = lean_unsigned_to_nat(1u); -x_47 = lean_nat_add(x_9, x_46); -x_48 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg(x_5, x_10, x_11, x_4, x_12, x_47, x_45, x_21, x_3, x_14, x_15, x_16, x_17, x_18, x_19, x_42); -return x_48; -} -else +lean_object* x_106; +x_106 = lean_ctor_get(x_1, 8); +lean_inc(x_106); +lean_dec(x_1); +if (lean_obj_tag(x_106) == 0) { -uint8_t x_49; -lean_dec(x_31); -lean_dec(x_23); -lean_dec(x_21); -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_8); -lean_dec(x_5); +lean_object* x_107; lean_object* x_108; uint8_t x_109; uint8_t x_110; lean_object* x_111; lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); -x_49 = !lean_is_exclusive(x_41); -if (x_49 == 0) -{ -return x_41; -} -else -{ -lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_50 = lean_ctor_get(x_41, 0); -x_51 = lean_ctor_get(x_41, 1); -lean_inc(x_51); -lean_inc(x_50); -lean_dec(x_41); -x_52 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_52, 0, x_50); -lean_ctor_set(x_52, 1, x_51); -return x_52; -} -} -} -else -{ -uint8_t x_53; -lean_dec(x_23); -lean_dec(x_21); -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); +x_107 = lean_ctor_get(x_105, 0); +lean_inc(x_107); +x_108 = lean_ctor_get(x_105, 1); +lean_inc(x_108); +lean_dec(x_105); +x_109 = 1; +x_110 = 1; +x_111 = l_Lean_Meta_mkForallFVars(x_107, x_99, x_102, x_109, x_110, x_5, x_6, x_7, x_8, x_108); lean_dec(x_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_53 = !lean_is_exclusive(x_30); -if (x_53 == 0) +if (lean_obj_tag(x_111) == 0) { -return x_30; +uint8_t x_112; +x_112 = !lean_is_exclusive(x_111); +if (x_112 == 0) +{ +lean_object* x_113; lean_object* x_114; lean_object* x_115; +x_113 = lean_ctor_get(x_111, 0); +lean_ctor_set(x_10, 0, x_113); +x_114 = lean_box(0); +x_115 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_115, 0, x_10); +lean_ctor_set(x_115, 1, x_114); +lean_ctor_set(x_111, 0, x_115); +return x_111; } else { -lean_object* x_54; lean_object* x_55; lean_object* x_56; -x_54 = lean_ctor_get(x_30, 0); -x_55 = lean_ctor_get(x_30, 1); -lean_inc(x_55); -lean_inc(x_54); -lean_dec(x_30); -x_56 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_56, 0, x_54); -lean_ctor_set(x_56, 1, x_55); -return x_56; -} +lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; +x_116 = lean_ctor_get(x_111, 0); +x_117 = lean_ctor_get(x_111, 1); +lean_inc(x_117); +lean_inc(x_116); +lean_dec(x_111); +lean_ctor_set(x_10, 0, x_116); +x_118 = lean_box(0); +x_119 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_119, 0, x_10); +lean_ctor_set(x_119, 1, x_118); +x_120 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_120, 0, x_119); +lean_ctor_set(x_120, 1, x_117); +return x_120; } } else { -uint8_t x_57; -lean_dec(x_21); -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_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_57 = !lean_is_exclusive(x_22); -if (x_57 == 0) +uint8_t x_121; +lean_free_object(x_10); +x_121 = !lean_is_exclusive(x_111); +if (x_121 == 0) { -return x_22; +return x_111; } else { -lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_58 = lean_ctor_get(x_22, 0); -x_59 = lean_ctor_get(x_22, 1); -lean_inc(x_59); -lean_inc(x_58); -lean_dec(x_22); -x_60 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_60, 0, x_58); -lean_ctor_set(x_60, 1, x_59); -return x_60; -} -} -} +lean_object* x_122; lean_object* x_123; lean_object* x_124; +x_122 = lean_ctor_get(x_111, 0); +x_123 = lean_ctor_get(x_111, 1); +lean_inc(x_123); +lean_inc(x_122); +lean_dec(x_111); +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_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18) { -_start: -{ -lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_19 = lean_unsigned_to_nat(1u); -x_20 = lean_nat_add(x_1, x_19); -x_21 = l_Lean_RBNode_insert___at_Lean_NameMap_insert___spec__1___rarg(x_2, x_3, x_4); -x_22 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg(x_5, x_6, x_7, x_8, x_9, x_20, x_11, x_21, x_10, x_12, x_13, x_14, x_15, x_16, x_17, x_18); -return x_22; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___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_object* x_13, lean_object* x_14, 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: +else { -lean_object* x_21; lean_object* x_22; uint8_t x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; -lean_inc(x_2); -lean_inc(x_1); -x_21 = l_Lean_Name_append(x_1, x_2); -x_22 = lean_box(0); -x_23 = 3; -lean_inc(x_13); -lean_inc(x_2); -x_24 = lean_alloc_ctor(0, 4, 1); -lean_ctor_set(x_24, 0, x_2); -lean_ctor_set(x_24, 1, x_21); -lean_ctor_set(x_24, 2, x_13); -lean_ctor_set(x_24, 3, x_22); -lean_ctor_set_uint8(x_24, sizeof(void*)*4, x_23); -x_25 = lean_array_push(x_3, x_24); -lean_inc(x_1); -lean_inc(x_13); -x_26 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__2___boxed), 18, 10); -lean_closure_set(x_26, 0, x_4); -lean_closure_set(x_26, 1, x_5); -lean_closure_set(x_26, 2, x_2); -lean_closure_set(x_26, 3, x_13); -lean_closure_set(x_26, 4, x_1); -lean_closure_set(x_26, 5, x_6); -lean_closure_set(x_26, 6, x_7); -lean_closure_set(x_26, 7, x_8); -lean_closure_set(x_26, 8, x_9); -lean_closure_set(x_26, 9, x_10); -x_27 = lean_unsigned_to_nat(0u); -x_28 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg(x_1, x_13, x_11, x_12, x_26, x_27, x_25, x_14, x_15, x_16, x_17, x_18, x_19, x_20); -return x_28; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19) { -_start: +lean_object* x_125; lean_object* x_126; uint8_t x_127; +x_125 = lean_ctor_get(x_105, 0); +lean_inc(x_125); +x_126 = lean_ctor_get(x_105, 1); +lean_inc(x_126); +lean_dec(x_105); +x_127 = !lean_is_exclusive(x_106); +if (x_127 == 0) { -lean_object* x_20; -lean_inc(x_18); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -x_20 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField(x_1, x_11, x_13, x_14, x_15, x_16, x_17, x_18, x_19); -if (lean_obj_tag(x_20) == 0) +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; +x_128 = lean_ctor_get(x_106, 0); +lean_inc(x_99); +lean_ctor_set(x_106, 0, x_99); +x_129 = lean_box(0); +x_130 = 1; +x_131 = lean_box(x_130); +x_132 = lean_box(x_130); +x_133 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTermEnsuringType___boxed), 12, 5); +lean_closure_set(x_133, 0, x_128); +lean_closure_set(x_133, 1, x_106); +lean_closure_set(x_133, 2, x_131); +lean_closure_set(x_133, 3, x_132); +lean_closure_set(x_133, 4, x_129); +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_134 = l_Lean_Elab_Term_withoutAutoBoundImplicit___rarg(x_133, x_3, x_4, x_5, x_6, x_7, x_8, x_126); +if (lean_obj_tag(x_134) == 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_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_unsigned_to_nat(1u); -x_24 = lean_nat_add(x_2, x_23); -x_25 = l_Lean_RBNode_insert___at_Lean_NameMap_insert___spec__1___rarg(x_3, x_4, x_21); -x_26 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg(x_5, x_6, x_7, x_8, x_9, x_24, x_10, x_25, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_22); -return x_26; -} -else +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_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_137 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_101, x_102, x_3, x_4, x_5, x_6, x_7, x_8, x_136); +if (lean_obj_tag(x_137) == 0) { -uint8_t x_27; -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_10); -lean_dec(x_9); +lean_object* x_138; uint8_t x_139; lean_object* x_140; +x_138 = lean_ctor_get(x_137, 1); +lean_inc(x_138); +lean_dec(x_137); +x_139 = 1; +lean_inc(x_125); +x_140 = l_Lean_Meta_mkForallFVars(x_125, x_99, x_102, x_130, x_139, x_5, x_6, x_7, x_8, x_138); +if (lean_obj_tag(x_140) == 0) +{ +lean_object* x_141; lean_object* x_142; lean_object* x_143; +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 = l_Lean_Meta_mkLambdaFVars(x_125, x_135, x_102, x_130, x_102, x_139, x_5, x_6, x_7, x_8, x_142); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_27 = !lean_is_exclusive(x_20); -if (x_27 == 0) +if (lean_obj_tag(x_143) == 0) { -return x_20; +uint8_t x_144; +x_144 = !lean_is_exclusive(x_143); +if (x_144 == 0) +{ +lean_object* x_145; lean_object* x_146; lean_object* x_147; +x_145 = lean_ctor_get(x_143, 0); +lean_ctor_set(x_10, 0, x_141); +x_146 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_146, 0, x_145); +x_147 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_147, 0, x_10); +lean_ctor_set(x_147, 1, x_146); +lean_ctor_set(x_143, 0, x_147); +return x_143; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_28 = lean_ctor_get(x_20, 0); -x_29 = lean_ctor_get(x_20, 1); -lean_inc(x_29); -lean_inc(x_28); -lean_dec(x_20); -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_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; +x_148 = lean_ctor_get(x_143, 0); +x_149 = lean_ctor_get(x_143, 1); +lean_inc(x_149); +lean_inc(x_148); +lean_dec(x_143); +lean_ctor_set(x_10, 0, x_141); +x_150 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_150, 0, x_148); +x_151 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_151, 0, x_10); +lean_ctor_set(x_151, 1, x_150); +x_152 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_152, 0, x_151); +lean_ctor_set(x_152, 1, x_149); +return x_152; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19) { -_start: +else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_20 = lean_unsigned_to_nat(1u); -x_21 = lean_nat_add(x_1, x_20); -x_22 = l_Lean_RBNode_insert___at_Lean_NameMap_insert___spec__1___rarg(x_2, x_3, x_4); -x_23 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg(x_5, x_6, x_7, x_8, x_9, x_21, x_10, x_22, x_11, x_13, x_14, x_15, x_16, x_17, x_18, x_19); -return x_23; -} -} -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__1() { -_start: +uint8_t x_153; +lean_dec(x_141); +lean_free_object(x_10); +x_153 = !lean_is_exclusive(x_143); +if (x_153 == 0) { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("_private.Lean.Elab.Structure.0.Lean.Elab.Command.copyNewFieldsFrom.copyFields.copy", 82, 82); -return x_1; -} +return x_143; } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__2() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__1; -x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__1; -x_3 = lean_unsigned_to_nat(409u); -x_4 = lean_unsigned_to_nat(86u); -x_5 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__3; -x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); -return x_6; -} +lean_object* x_154; lean_object* x_155; lean_object* x_156; +x_154 = lean_ctor_get(x_143, 0); +x_155 = lean_ctor_get(x_143, 1); +lean_inc(x_155); +lean_inc(x_154); +lean_dec(x_143); +x_156 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_156, 0, x_154); +lean_ctor_set(x_156, 1, x_155); +return x_156; } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("parent field type mismatch, field '", 35, 35); -return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__4() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__3; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__5() { -_start: +uint8_t x_157; +lean_dec(x_135); +lean_dec(x_125); +lean_free_object(x_10); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_157 = !lean_is_exclusive(x_140); +if (x_157 == 0) { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("' from parent '", 15, 15); -return x_1; -} +return x_140; } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__6() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__5; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} +lean_object* x_158; lean_object* x_159; lean_object* x_160; +x_158 = lean_ctor_get(x_140, 0); +x_159 = lean_ctor_get(x_140, 1); +lean_inc(x_159); +lean_inc(x_158); +lean_dec(x_140); +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; } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__7() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("' ", 2, 2); -return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__8() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__7; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: -{ -lean_object* x_17; uint8_t x_18; -x_17 = lean_array_get_size(x_5); -x_18 = lean_nat_dec_lt(x_6, x_17); -lean_dec(x_17); -if (x_18 == 0) -{ -lean_object* x_19; +uint8_t x_161; +lean_dec(x_135); +lean_dec(x_125); +lean_dec(x_99); +lean_free_object(x_10); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_2); -lean_dec(x_1); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_10); -lean_inc(x_9); -x_19 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_processOveriddenDefaultValues(x_7, x_8, x_9, x_4, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_19) == 0) +x_161 = !lean_is_exclusive(x_137); +if (x_161 == 0) { -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_19, 1); -lean_inc(x_21); -lean_dec(x_19); -x_22 = lean_apply_10(x_3, x_20, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_21); -return x_22; +return x_137; } else { -uint8_t x_23; -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); +lean_object* x_162; lean_object* x_163; lean_object* x_164; +x_162 = lean_ctor_get(x_137, 0); +x_163 = lean_ctor_get(x_137, 1); +lean_inc(x_163); +lean_inc(x_162); +lean_dec(x_137); +x_164 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_164, 0, x_162); +lean_ctor_set(x_164, 1, x_163); +return x_164; +} +} +} +else +{ +uint8_t x_165; +lean_dec(x_125); +lean_dec(x_99); +lean_free_object(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); -x_23 = !lean_is_exclusive(x_19); -if (x_23 == 0) +x_165 = !lean_is_exclusive(x_134); +if (x_165 == 0) { -return x_19; +return x_134; } else { -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_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; +lean_object* x_166; lean_object* x_167; lean_object* x_168; +x_166 = lean_ctor_get(x_134, 0); +x_167 = lean_ctor_get(x_134, 1); +lean_inc(x_167); +lean_inc(x_166); +lean_dec(x_134); +x_168 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_168, 0, x_166); +lean_ctor_set(x_168, 1, x_167); +return x_168; } } } else { -lean_object* x_27; lean_object* x_28; -x_27 = lean_array_fget(x_5, x_6); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_27); -lean_inc(x_2); +lean_object* x_169; lean_object* x_170; lean_object* x_171; uint8_t x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; +x_169 = lean_ctor_get(x_106, 0); +lean_inc(x_169); +lean_dec(x_106); +lean_inc(x_99); +x_170 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_170, 0, x_99); +x_171 = lean_box(0); +x_172 = 1; +x_173 = lean_box(x_172); +x_174 = lean_box(x_172); +x_175 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTermEnsuringType___boxed), 12, 5); +lean_closure_set(x_175, 0, x_169); +lean_closure_set(x_175, 1, x_170); +lean_closure_set(x_175, 2, x_173); +lean_closure_set(x_175, 3, x_174); +lean_closure_set(x_175, 4, x_171); +lean_inc(x_8); lean_inc(x_7); -x_28 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType(x_7, x_2, x_27, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_28) == 0) +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_176 = l_Lean_Elab_Term_withoutAutoBoundImplicit___rarg(x_175, x_3, x_4, x_5, x_6, x_7, x_8, x_126); +if (lean_obj_tag(x_176) == 0) { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_28, 0); -lean_inc(x_29); -x_30 = lean_ctor_get(x_28, 1); -lean_inc(x_30); -lean_dec(x_28); -x_31 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f(x_7, x_27); -if (lean_obj_tag(x_31) == 0) +lean_object* x_177; lean_object* x_178; lean_object* 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); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_179 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_101, x_102, x_3, x_4, x_5, x_6, x_7, x_8, x_178); +if (lean_obj_tag(x_179) == 0) { -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_32 = lean_st_ref_get(x_15, x_30); -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_dec(x_33); -lean_inc(x_27); -lean_inc(x_4); -x_36 = l_Lean_getFieldInfo_x3f(x_35, x_4, x_27); -lean_dec(x_35); -if (lean_obj_tag(x_36) == 0) +lean_object* x_180; uint8_t x_181; lean_object* x_182; +x_180 = lean_ctor_get(x_179, 1); +lean_inc(x_180); +lean_dec(x_179); +x_181 = 1; +lean_inc(x_125); +x_182 = l_Lean_Meta_mkForallFVars(x_125, x_99, x_102, x_172, x_181, x_5, x_6, x_7, x_8, x_180); +if (lean_obj_tag(x_182) == 0) { -lean_object* x_37; lean_object* x_38; -lean_dec(x_29); -lean_dec(x_27); -lean_dec(x_9); +lean_object* x_183; lean_object* x_184; lean_object* x_185; +x_183 = lean_ctor_get(x_182, 0); +lean_inc(x_183); +x_184 = lean_ctor_get(x_182, 1); +lean_inc(x_184); +lean_dec(x_182); +x_185 = l_Lean_Meta_mkLambdaFVars(x_125, x_177, x_102, x_172, x_102, x_181, x_5, x_6, x_7, x_8, x_184); lean_dec(x_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_37 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__2; -x_38 = l_panic___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___spec__1___rarg(x_37, x_10, x_11, x_12, x_13, x_14, x_15, x_34); -return x_38; +if (lean_obj_tag(x_185) == 0) +{ +lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; +x_186 = lean_ctor_get(x_185, 0); +lean_inc(x_186); +x_187 = lean_ctor_get(x_185, 1); +lean_inc(x_187); +if (lean_is_exclusive(x_185)) { + lean_ctor_release(x_185, 0); + lean_ctor_release(x_185, 1); + x_188 = x_185; +} else { + lean_dec_ref(x_185); + x_188 = lean_box(0); +} +lean_ctor_set(x_10, 0, x_183); +x_189 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_189, 0, x_186); +x_190 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_190, 0, x_10); +lean_ctor_set(x_190, 1, x_189); +if (lean_is_scalar(x_188)) { + x_191 = lean_alloc_ctor(0, 2, 0); +} else { + x_191 = x_188; +} +lean_ctor_set(x_191, 0, x_190); +lean_ctor_set(x_191, 1, x_187); +return x_191; } else { -lean_object* x_39; lean_object* x_40; -x_39 = lean_ctor_get(x_36, 0); -lean_inc(x_39); -lean_dec(x_36); -x_40 = lean_ctor_get(x_39, 2); -lean_inc(x_40); -if (lean_obj_tag(x_40) == 0) -{ -lean_object* x_41; uint8_t x_42; lean_object* x_43; uint8_t x_44; lean_object* x_45; -x_41 = lean_ctor_get(x_39, 1); -lean_inc(x_41); -x_42 = lean_ctor_get_uint8(x_39, sizeof(void*)*4); -lean_inc(x_27); -x_43 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__1___boxed), 20, 12); -lean_closure_set(x_43, 0, x_8); -lean_closure_set(x_43, 1, x_27); -lean_closure_set(x_43, 2, x_9); -lean_closure_set(x_43, 3, x_4); -lean_closure_set(x_43, 4, x_1); -lean_closure_set(x_43, 5, x_39); -lean_closure_set(x_43, 6, x_41); -lean_closure_set(x_43, 7, x_7); -lean_closure_set(x_43, 8, x_6); -lean_closure_set(x_43, 9, x_2); -lean_closure_set(x_43, 10, x_3); -lean_closure_set(x_43, 11, x_5); -x_44 = 0; -x_45 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__1___rarg(x_27, x_42, x_29, x_43, x_44, x_10, x_11, x_12, x_13, x_14, x_15, x_34); -return x_45; +lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; +lean_dec(x_183); +lean_free_object(x_10); +x_192 = lean_ctor_get(x_185, 0); +lean_inc(x_192); +x_193 = lean_ctor_get(x_185, 1); +lean_inc(x_193); +if (lean_is_exclusive(x_185)) { + lean_ctor_release(x_185, 0); + lean_ctor_release(x_185, 1); + x_194 = x_185; +} else { + lean_dec_ref(x_185); + x_194 = lean_box(0); +} +if (lean_is_scalar(x_194)) { + x_195 = lean_alloc_ctor(1, 2, 0); +} else { + x_195 = x_194; +} +lean_ctor_set(x_195, 0, x_192); +lean_ctor_set(x_195, 1, x_193); +return x_195; +} } else { -lean_object* x_46; uint8_t x_47; lean_object* x_48; -lean_dec(x_40); -x_46 = lean_ctor_get(x_39, 0); -lean_inc(x_46); -x_47 = lean_ctor_get_uint8(x_39, sizeof(void*)*4); -lean_dec(x_39); -x_48 = l_Lean_Meta_getStructureName(x_29, x_12, x_13, x_14, x_15, x_34); -if (lean_obj_tag(x_48) == 0) -{ -lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_49 = lean_ctor_get(x_48, 0); -lean_inc(x_49); -x_50 = lean_ctor_get(x_48, 1); -lean_inc(x_50); -lean_dec(x_48); -lean_inc(x_49); -x_51 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f(x_7, x_49, x_14, x_15, x_50); -x_52 = lean_ctor_get(x_51, 0); -lean_inc(x_52); -if (lean_obj_tag(x_52) == 0) -{ -lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; uint8_t x_58; lean_object* x_59; lean_object* x_60; uint8_t x_61; lean_object* x_62; -lean_dec(x_27); -x_53 = lean_ctor_get(x_51, 1); -lean_inc(x_53); -lean_dec(x_51); -x_54 = lean_st_ref_get(x_15, x_53); -x_55 = lean_ctor_get(x_54, 0); -lean_inc(x_55); -x_56 = lean_ctor_get(x_54, 1); -lean_inc(x_56); -lean_dec(x_54); -x_57 = lean_ctor_get(x_55, 0); -lean_inc(x_57); -lean_dec(x_55); -x_58 = 1; -lean_inc(x_49); -x_59 = l_Lean_getStructureFieldsFlattened(x_57, x_49, x_58); -lean_dec(x_57); -lean_inc(x_46); -x_60 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__3___boxed), 20, 12); -lean_closure_set(x_60, 0, x_1); -lean_closure_set(x_60, 1, x_46); -lean_closure_set(x_60, 2, x_7); -lean_closure_set(x_60, 3, x_6); -lean_closure_set(x_60, 4, x_8); -lean_closure_set(x_60, 5, x_2); -lean_closure_set(x_60, 6, x_3); -lean_closure_set(x_60, 7, x_4); -lean_closure_set(x_60, 8, x_5); -lean_closure_set(x_60, 9, x_9); -lean_closure_set(x_60, 10, x_49); -lean_closure_set(x_60, 11, x_59); -x_61 = 0; -x_62 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__1___rarg(x_46, x_47, x_29, x_60, x_61, x_10, x_11, x_12, x_13, x_14, x_15, x_56); -return x_62; +lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; +lean_dec(x_177); +lean_dec(x_125); +lean_free_object(x_10); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_196 = lean_ctor_get(x_182, 0); +lean_inc(x_196); +x_197 = lean_ctor_get(x_182, 1); +lean_inc(x_197); +if (lean_is_exclusive(x_182)) { + lean_ctor_release(x_182, 0); + lean_ctor_release(x_182, 1); + x_198 = x_182; +} else { + lean_dec_ref(x_182); + 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_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; -lean_dec(x_52); -lean_dec(x_46); -x_63 = lean_ctor_get(x_51, 1); -lean_inc(x_63); -lean_dec(x_51); -x_64 = lean_box(0); -x_65 = l_Lean_RBNode_insert___at_Lean_NameSet_insert___spec__1(x_9, x_49, x_64); -lean_inc(x_1); -lean_inc(x_29); -x_66 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__4___boxed), 19, 9); -lean_closure_set(x_66, 0, x_29); -lean_closure_set(x_66, 1, x_6); -lean_closure_set(x_66, 2, x_8); -lean_closure_set(x_66, 3, x_27); -lean_closure_set(x_66, 4, x_1); -lean_closure_set(x_66, 5, x_2); -lean_closure_set(x_66, 6, x_3); -lean_closure_set(x_66, 7, x_4); -lean_closure_set(x_66, 8, x_5); -x_67 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields___rarg(x_1, x_7, x_65, x_29, x_66, x_10, x_11, x_12, x_13, x_14, x_15, x_63); -return x_67; +lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; +lean_dec(x_177); +lean_dec(x_125); +lean_dec(x_99); +lean_free_object(x_10); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_200 = lean_ctor_get(x_179, 0); +lean_inc(x_200); +x_201 = lean_ctor_get(x_179, 1); +lean_inc(x_201); +if (lean_is_exclusive(x_179)) { + lean_ctor_release(x_179, 0); + lean_ctor_release(x_179, 1); + x_202 = x_179; +} else { + lean_dec_ref(x_179); + 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 { -uint8_t x_68; -lean_dec(x_46); -lean_dec(x_29); -lean_dec(x_27); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); +lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; +lean_dec(x_125); +lean_dec(x_99); +lean_free_object(x_10); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_68 = !lean_is_exclusive(x_48); -if (x_68 == 0) -{ -return x_48; +x_204 = lean_ctor_get(x_176, 0); +lean_inc(x_204); +x_205 = lean_ctor_get(x_176, 1); +lean_inc(x_205); +if (lean_is_exclusive(x_176)) { + lean_ctor_release(x_176, 0); + lean_ctor_release(x_176, 1); + x_206 = x_176; +} else { + lean_dec_ref(x_176); + x_206 = lean_box(0); } -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; +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; } } } } else { -lean_object* x_72; lean_object* x_73; lean_object* x_74; -x_72 = lean_ctor_get(x_31, 0); -lean_inc(x_72); -lean_dec(x_31); -x_73 = lean_ctor_get(x_72, 2); -lean_inc(x_73); -lean_dec(x_72); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_73); -x_74 = lean_infer_type(x_73, x_12, x_13, x_14, x_15, x_30); -if (lean_obj_tag(x_74) == 0) -{ -lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_75 = lean_ctor_get(x_74, 0); -lean_inc(x_75); -x_76 = lean_ctor_get(x_74, 1); -lean_inc(x_76); -lean_dec(x_74); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_75); -lean_inc(x_29); -x_77 = l_Lean_Meta_isExprDefEq(x_29, x_75, x_12, x_13, x_14, x_15, x_76); -if (lean_obj_tag(x_77) == 0) -{ -lean_object* x_78; uint8_t x_79; -x_78 = lean_ctor_get(x_77, 0); -lean_inc(x_78); -x_79 = lean_unbox(x_78); -lean_dec(x_78); -if (x_79 == 0) -{ -lean_object* x_80; lean_object* x_81; -lean_dec(x_73); -lean_dec(x_9); +uint8_t x_208; +lean_dec(x_99); +lean_free_object(x_10); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); lean_dec(x_1); -x_80 = lean_ctor_get(x_77, 1); -lean_inc(x_80); -lean_dec(x_77); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -x_81 = l_Lean_Meta_mkHasTypeButIsExpectedMsg(x_29, x_75, x_12, x_13, x_14, x_15, x_80); -if (lean_obj_tag(x_81) == 0) -{ -lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; uint8_t x_97; -x_82 = lean_ctor_get(x_81, 0); -lean_inc(x_82); -x_83 = lean_ctor_get(x_81, 1); -lean_inc(x_83); -lean_dec(x_81); -x_84 = l_Lean_MessageData_ofName(x_27); -x_85 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__4; -x_86 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_86, 0, x_85); -lean_ctor_set(x_86, 1, x_84); -x_87 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__6; -x_88 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_88, 0, x_86); -lean_ctor_set(x_88, 1, x_87); -x_89 = l_Lean_MessageData_ofName(x_4); -x_90 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_90, 0, x_88); -lean_ctor_set(x_90, 1, x_89); -x_91 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__8; -x_92 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_92, 0, x_90); -lean_ctor_set(x_92, 1, x_91); -x_93 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_93, 0, x_92); -lean_ctor_set(x_93, 1, x_82); -x_94 = l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__4; -x_95 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_95, 0, x_93); -lean_ctor_set(x_95, 1, x_94); -x_96 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_95, x_10, x_11, x_12, x_13, x_14, x_15, x_83); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -x_97 = !lean_is_exclusive(x_96); -if (x_97 == 0) +x_208 = !lean_is_exclusive(x_105); +if (x_208 == 0) { -return x_96; +return x_105; } else { -lean_object* x_98; lean_object* x_99; lean_object* x_100; -x_98 = lean_ctor_get(x_96, 0); -x_99 = lean_ctor_get(x_96, 1); -lean_inc(x_99); -lean_inc(x_98); -lean_dec(x_96); -x_100 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_100, 0, x_98); -lean_ctor_set(x_100, 1, x_99); -return x_100; +lean_object* x_209; lean_object* x_210; lean_object* x_211; +x_209 = lean_ctor_get(x_105, 0); +x_210 = lean_ctor_get(x_105, 1); +lean_inc(x_210); +lean_inc(x_209); +lean_dec(x_105); +x_211 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_211, 0, x_209); +lean_ctor_set(x_211, 1, x_210); +return x_211; } } -else -{ -uint8_t x_101; -lean_dec(x_27); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_4); -x_101 = !lean_is_exclusive(x_81); -if (x_101 == 0) -{ -return x_81; } else { -lean_object* x_102; lean_object* x_103; lean_object* x_104; -x_102 = lean_ctor_get(x_81, 0); -x_103 = lean_ctor_get(x_81, 1); -lean_inc(x_103); -lean_inc(x_102); -lean_dec(x_81); -x_104 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_104, 0, x_102); -lean_ctor_set(x_104, 1, x_103); -return x_104; -} -} -} -else -{ -lean_object* x_105; lean_object* x_106; lean_object* x_107; -lean_dec(x_75); -lean_dec(x_29); -x_105 = lean_ctor_get(x_77, 1); -lean_inc(x_105); -lean_dec(x_77); -x_106 = lean_box(0); -x_107 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__5(x_6, x_8, x_27, x_73, x_1, x_2, x_3, x_4, x_5, x_7, x_9, x_106, x_10, x_11, x_12, x_13, x_14, x_15, x_105); -lean_dec(x_6); -return x_107; -} -} -else -{ -uint8_t x_108; -lean_dec(x_75); -lean_dec(x_73); -lean_dec(x_29); -lean_dec(x_27); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); +uint8_t x_212; +lean_dec(x_99); +lean_free_object(x_10); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); lean_dec(x_1); -x_108 = !lean_is_exclusive(x_77); -if (x_108 == 0) +x_212 = !lean_is_exclusive(x_103); +if (x_212 == 0) { -return x_77; +return x_103; } else { -lean_object* x_109; lean_object* x_110; lean_object* x_111; -x_109 = lean_ctor_get(x_77, 0); -x_110 = lean_ctor_get(x_77, 1); -lean_inc(x_110); -lean_inc(x_109); -lean_dec(x_77); -x_111 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_111, 0, x_109); -lean_ctor_set(x_111, 1, x_110); -return x_111; +lean_object* x_213; lean_object* x_214; lean_object* x_215; +x_213 = lean_ctor_get(x_103, 0); +x_214 = lean_ctor_get(x_103, 1); +lean_inc(x_214); +lean_inc(x_213); +lean_dec(x_103); +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; } } } else { -uint8_t x_112; -lean_dec(x_73); -lean_dec(x_29); -lean_dec(x_27); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); +uint8_t x_216; +lean_free_object(x_10); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); lean_dec(x_1); -x_112 = !lean_is_exclusive(x_74); -if (x_112 == 0) +x_216 = !lean_is_exclusive(x_98); +if (x_216 == 0) { -return x_74; +return x_98; } else { -lean_object* x_113; lean_object* x_114; lean_object* x_115; -x_113 = lean_ctor_get(x_74, 0); -x_114 = lean_ctor_get(x_74, 1); -lean_inc(x_114); -lean_inc(x_113); -lean_dec(x_74); -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_217; lean_object* x_218; lean_object* x_219; +x_217 = lean_ctor_get(x_98, 0); +x_218 = lean_ctor_get(x_98, 1); +lean_inc(x_218); +lean_inc(x_217); +lean_dec(x_98); +x_219 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_219, 0, x_217); +lean_ctor_set(x_219, 1, x_218); +return x_219; } } } else { -uint8_t x_116; -lean_dec(x_27); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); +lean_object* x_220; lean_object* x_221; +x_220 = lean_ctor_get(x_10, 0); +lean_inc(x_220); lean_dec(x_10); -lean_dec(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_221 = l_Lean_Elab_Term_elabType(x_220, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_221) == 0) +{ +lean_object* x_222; lean_object* x_223; uint8_t x_224; uint8_t x_225; lean_object* x_226; +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 = 1; +x_225 = 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_226 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_224, x_225, x_3, x_4, x_5, x_6, x_7, x_8, x_223); +if (lean_obj_tag(x_226) == 0) +{ +lean_object* x_227; lean_object* x_228; +x_227 = lean_ctor_get(x_226, 1); +lean_inc(x_227); +lean_dec(x_226); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_3); +x_228 = l_Lean_Elab_Term_addAutoBoundImplicits(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_227); +if (lean_obj_tag(x_228) == 0) +{ +lean_object* x_229; +x_229 = lean_ctor_get(x_1, 8); +lean_inc(x_229); +lean_dec(x_1); +if (lean_obj_tag(x_229) == 0) +{ +lean_object* x_230; lean_object* x_231; uint8_t x_232; uint8_t x_233; lean_object* x_234; +lean_dec(x_4); +lean_dec(x_3); +x_230 = lean_ctor_get(x_228, 0); +lean_inc(x_230); +x_231 = lean_ctor_get(x_228, 1); +lean_inc(x_231); +lean_dec(x_228); +x_232 = 1; +x_233 = 1; +x_234 = l_Lean_Meta_mkForallFVars(x_230, x_222, x_225, x_232, x_233, x_5, x_6, x_7, x_8, x_231); lean_dec(x_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_116 = !lean_is_exclusive(x_28); -if (x_116 == 0) +if (lean_obj_tag(x_234) == 0) { -return x_28; +lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; +x_235 = lean_ctor_get(x_234, 0); +lean_inc(x_235); +x_236 = lean_ctor_get(x_234, 1); +lean_inc(x_236); +if (lean_is_exclusive(x_234)) { + lean_ctor_release(x_234, 0); + lean_ctor_release(x_234, 1); + x_237 = x_234; +} else { + lean_dec_ref(x_234); + x_237 = lean_box(0); +} +x_238 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_238, 0, x_235); +x_239 = lean_box(0); +x_240 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_240, 0, x_238); +lean_ctor_set(x_240, 1, x_239); +if (lean_is_scalar(x_237)) { + x_241 = lean_alloc_ctor(0, 2, 0); +} else { + x_241 = x_237; +} +lean_ctor_set(x_241, 0, x_240); +lean_ctor_set(x_241, 1, x_236); +return x_241; } else { -lean_object* x_117; lean_object* x_118; lean_object* x_119; -x_117 = lean_ctor_get(x_28, 0); -x_118 = lean_ctor_get(x_28, 1); -lean_inc(x_118); -lean_inc(x_117); -lean_dec(x_28); -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_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; +x_242 = lean_ctor_get(x_234, 0); +lean_inc(x_242); +x_243 = lean_ctor_get(x_234, 1); +lean_inc(x_243); +if (lean_is_exclusive(x_234)) { + lean_ctor_release(x_234, 0); + lean_ctor_release(x_234, 1); + x_244 = x_234; +} else { + lean_dec_ref(x_234); + x_244 = lean_box(0); } +if (lean_is_scalar(x_244)) { + x_245 = lean_alloc_ctor(1, 2, 0); +} else { + x_245 = x_244; } +lean_ctor_set(x_245, 0, x_242); +lean_ctor_set(x_245, 1, x_243); +return x_245; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy(lean_object* x_1) { -_start: +else { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg), 16, 0); -return x_2; +lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; uint8_t x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; +x_246 = lean_ctor_get(x_228, 0); +lean_inc(x_246); +x_247 = lean_ctor_get(x_228, 1); +lean_inc(x_247); +lean_dec(x_228); +x_248 = lean_ctor_get(x_229, 0); +lean_inc(x_248); +if (lean_is_exclusive(x_229)) { + lean_ctor_release(x_229, 0); + x_249 = x_229; +} else { + lean_dec_ref(x_229); + x_249 = lean_box(0); } -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___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]; -lean_object* x_20 = _args[19]; -_start: -{ -lean_object* x_21; -x_21 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20); -lean_dec(x_9); -return x_21; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__2___boxed(lean_object** _args) { -lean_object* x_1 = _args[0]; -lean_object* x_2 = _args[1]; -lean_object* x_3 = _args[2]; -lean_object* x_4 = _args[3]; -lean_object* x_5 = _args[4]; -lean_object* x_6 = _args[5]; -lean_object* x_7 = _args[6]; -lean_object* x_8 = _args[7]; -lean_object* x_9 = _args[8]; -lean_object* x_10 = _args[9]; -lean_object* x_11 = _args[10]; -lean_object* x_12 = _args[11]; -lean_object* x_13 = _args[12]; -lean_object* x_14 = _args[13]; -lean_object* x_15 = _args[14]; -lean_object* x_16 = _args[15]; -lean_object* x_17 = _args[16]; -lean_object* x_18 = _args[17]; -_start: -{ -lean_object* x_19; -x_19 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18); -lean_dec(x_1); -return x_19; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___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]; -lean_object* x_18 = _args[17]; -lean_object* x_19 = _args[18]; -lean_object* x_20 = _args[19]; -_start: -{ -lean_object* x_21; -x_21 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20); -return x_21; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__4___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_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19); -lean_dec(x_11); -lean_dec(x_2); -return x_20; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___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]; -lean_object* x_18 = _args[17]; -lean_object* x_19 = _args[18]; -_start: -{ -lean_object* x_20; -x_20 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19); -lean_dec(x_12); -lean_dec(x_1); -return x_20; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom___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) { -_start: -{ -lean_object* x_12; -x_12 = lean_apply_8(x_1, x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -return x_12; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom___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; -x_12 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom___rarg___lambda__1___boxed), 11, 1); -lean_closure_set(x_12, 0, x_4); -x_13 = l_Lean_NameSet_empty; -x_14 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields___rarg(x_1, x_2, x_13, x_3, x_12, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -return x_14; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom___rarg), 11, 0); -return x_2; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -lean_object* x_12; -x_12 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_4); -lean_dec(x_3); -return x_12; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkToParentName_go(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_3); -lean_inc(x_2); -x_4 = lean_name_append_index_after(x_2, x_3); -lean_inc(x_1); -lean_inc(x_4); -x_5 = lean_apply_1(x_1, x_4); -x_6 = lean_unbox(x_5); -lean_dec(x_5); -if (x_6 == 0) -{ -lean_object* x_7; lean_object* x_8; -lean_dec(x_4); -x_7 = lean_unsigned_to_nat(1u); -x_8 = lean_nat_add(x_3, x_7); -lean_dec(x_3); -x_3 = x_8; -goto _start; -} -else -{ -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_4; -} -} -} -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkToParentName___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("to", 2, 2); -return x_1; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkToParentName(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; uint8_t x_10; -x_3 = lean_erase_macro_scopes(x_1); -x_4 = l_Lean_Name_getString_x21(x_3); -lean_dec(x_3); -x_5 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkToParentName___closed__1; -x_6 = lean_string_append(x_5, x_4); -lean_dec(x_4); -x_7 = lean_box(0); -x_8 = l_Lean_Name_str___override(x_7, x_6); -lean_inc(x_2); -lean_inc(x_8); -x_9 = lean_apply_1(x_2, x_8); -x_10 = lean_unbox(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 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkToParentName_go(x_2, x_8, x_11); -return x_12; -} -else -{ -lean_dec(x_2); -return x_8; -} -} -} -LEAN_EXPORT uint8_t l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -uint8_t x_4; -x_4 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_containsFieldName(x_1, x_3); -if (x_4 == 0) -{ -uint8_t x_5; -x_5 = l_Array_contains___at_Lean_findField_x3f___spec__1(x_2, x_3); -if (x_5 == 0) -{ -uint8_t x_6; -x_6 = 1; -return x_6; -} -else -{ -uint8_t x_7; -x_7 = 0; -return x_7; -} -} -else -{ -uint8_t x_8; -x_8 = 0; -return x_8; -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_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, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_unsigned_to_nat(1u); -x_14 = lean_nat_add(x_1, x_13); -x_15 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg(x_2, x_3, x_14, x_5, x_4, 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_Structure_0__Lean_Elab_Command_withParents_go___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, 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; uint8_t 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_1, 4); -lean_inc(x_17); -lean_inc(x_2); -lean_inc(x_17); -x_18 = l_Lean_Name_append(x_17, x_2); -x_19 = lean_box(0); -x_20 = 3; -lean_inc(x_9); -x_21 = lean_alloc_ctor(0, 4, 1); -lean_ctor_set(x_21, 0, x_2); -lean_ctor_set(x_21, 1, x_18); -lean_ctor_set(x_21, 2, x_9); -lean_ctor_set(x_21, 3, x_19); -lean_ctor_set_uint8(x_21, sizeof(void*)*4, x_20); -x_22 = lean_array_push(x_3, x_21); -x_23 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___lambda__2___boxed), 12, 4); -lean_closure_set(x_23, 0, x_4); -lean_closure_set(x_23, 1, x_1); -lean_closure_set(x_23, 2, x_5); -lean_closure_set(x_23, 3, x_6); -x_24 = lean_unsigned_to_nat(0u); -x_25 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg(x_17, x_9, x_7, x_8, x_23, x_24, x_22, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -return x_25; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { -_start: -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_14 = lean_unsigned_to_nat(1u); -x_15 = lean_nat_add(x_1, x_14); -x_16 = lean_array_push(x_2, x_3); -x_17 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg(x_4, x_5, x_15, x_6, x_16, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -return x_17; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { -_start: -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = lean_ctor_get(x_1, 4); -lean_inc(x_15); -lean_inc(x_4); -x_16 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___lambda__4___boxed), 13, 5); -lean_closure_set(x_16, 0, x_2); -lean_closure_set(x_16, 1, x_3); -lean_closure_set(x_16, 2, x_4); -lean_closure_set(x_16, 3, x_1); -lean_closure_set(x_16, 4, x_5); -x_17 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom___rarg(x_15, x_6, x_4, x_16, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -return x_17; -} -} -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_Elab_Command_structureDiamondWarning; -return x_1; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___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_13; lean_object* x_14; uint8_t x_15; -x_13 = lean_ctor_get(x_1, 7); -lean_inc(x_13); -x_14 = lean_array_get_size(x_13); -x_15 = lean_nat_dec_lt(x_3, x_14); -lean_dec(x_14); -if (x_15 == 0) -{ -lean_object* x_16; -lean_dec(x_13); -lean_dec(x_3); -lean_dec(x_1); -x_16 = lean_apply_9(x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -return x_16; -} -else -{ -lean_object* x_17; lean_object* x_18; uint8_t x_19; -x_17 = lean_array_fget(x_13, x_3); -lean_dec(x_13); -lean_inc(x_17); -x_18 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabType), 8, 1); -lean_closure_set(x_18, 0, x_17); -x_19 = !lean_is_exclusive(x_10); -if (x_19 == 0) -{ -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_10, 2); -x_21 = lean_ctor_get(x_10, 5); -x_22 = l_Lean_replaceRef(x_17, x_21); -lean_dec(x_21); -lean_dec(x_17); -lean_inc(x_20); -lean_ctor_set(x_10, 5, x_22); -x_23 = 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_24 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_withSynthesizeImp___rarg(x_18, x_23, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_24) == 0) -{ -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_24, 0); -lean_inc(x_25); -x_26 = lean_ctor_get(x_24, 1); -lean_inc(x_26); -lean_dec(x_24); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -x_27 = lean_whnf(x_25, x_8, x_9, x_10, x_11, x_26); -if (lean_obj_tag(x_27) == 0) -{ -lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_28 = lean_ctor_get(x_27, 0); -lean_inc(x_28); -x_29 = lean_ctor_get(x_27, 1); -lean_inc(x_29); -lean_dec(x_27); -x_30 = l_Lean_Meta_getStructureName(x_28, x_8, x_9, x_10, x_11, 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; -x_31 = lean_ctor_get(x_30, 0); -lean_inc(x_31); -x_32 = lean_ctor_get(x_30, 1); -lean_inc(x_32); -lean_dec(x_30); -lean_inc(x_31); -x_33 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f(x_4, x_31, x_10, x_11, x_32); -x_34 = lean_ctor_get(x_33, 0); -lean_inc(x_34); -if (lean_obj_tag(x_34) == 0) -{ -lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; lean_object* x_45; -lean_dec(x_20); -x_35 = lean_ctor_get(x_33, 1); -lean_inc(x_35); -lean_dec(x_33); -x_36 = lean_st_ref_get(x_11, 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); -x_39 = lean_ctor_get(x_37, 0); -lean_inc(x_39); -lean_dec(x_37); -x_40 = 1; -lean_inc(x_31); -x_41 = l_Lean_getStructureFieldsFlattened(x_39, x_31, x_40); -lean_inc(x_41); -lean_inc(x_4); -x_42 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___lambda__1___boxed), 3, 2); -lean_closure_set(x_42, 0, x_4); -lean_closure_set(x_42, 1, x_41); -lean_inc(x_31); -x_43 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkToParentName(x_31, x_42); -x_44 = lean_ctor_get_uint8(x_1, sizeof(void*)*11); -lean_inc(x_31); -lean_inc(x_43); -x_45 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___lambda__3), 16, 8); -lean_closure_set(x_45, 0, x_1); -lean_closure_set(x_45, 1, x_43); -lean_closure_set(x_45, 2, x_4); -lean_closure_set(x_45, 3, x_3); -lean_closure_set(x_45, 4, x_2); -lean_closure_set(x_45, 5, x_5); -lean_closure_set(x_45, 6, x_31); -lean_closure_set(x_45, 7, x_41); -if (x_44 == 0) -{ -uint8_t x_46; uint8_t x_47; lean_object* x_48; -lean_dec(x_39); -lean_dec(x_31); -x_46 = 0; -x_47 = 0; -x_48 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__1___rarg(x_43, x_46, x_28, x_45, x_47, x_6, x_7, x_8, x_9, x_10, x_11, x_38); -return x_48; -} -else -{ -uint8_t x_49; -x_49 = lean_is_class(x_39, x_31); -if (x_49 == 0) -{ -uint8_t x_50; uint8_t x_51; lean_object* x_52; -x_50 = 0; -x_51 = 0; -x_52 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__1___rarg(x_43, x_50, x_28, x_45, x_51, x_6, x_7, x_8, x_9, x_10, x_11, x_38); -return x_52; -} -else -{ -uint8_t x_53; uint8_t x_54; lean_object* x_55; -x_53 = 3; -x_54 = 0; -x_55 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__1___rarg(x_43, x_53, x_28, x_45, x_54, x_6, x_7, x_8, x_9, x_10, x_11, x_38); -return x_55; -} -} -} -else -{ -lean_object* x_56; uint8_t x_57; -x_56 = lean_ctor_get(x_33, 1); -lean_inc(x_56); -lean_dec(x_33); -x_57 = !lean_is_exclusive(x_34); -if (x_57 == 0) -{ -lean_object* x_58; lean_object* x_59; uint8_t x_60; -x_58 = lean_ctor_get(x_34, 0); -x_59 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___closed__1; -x_60 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_20, x_59); -lean_dec(x_20); -if (x_60 == 0) -{ -lean_object* x_61; lean_object* x_62; -lean_free_object(x_34); -lean_dec(x_58); -lean_dec(x_31); -x_61 = lean_box(0); -x_62 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___lambda__5(x_1, x_3, x_5, x_28, x_2, x_4, x_61, x_6, x_7, x_8, x_9, x_10, x_11, x_56); -return x_62; -} -else -{ -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_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; -x_63 = 1; -x_64 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___closed__1; -x_65 = l_Lean_Name_toString(x_58, x_63, x_64); -x_66 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__1; -x_67 = lean_string_append(x_66, x_65); -lean_dec(x_65); -x_68 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__3; -x_69 = lean_string_append(x_67, x_68); -x_70 = l_Lean_Name_toString(x_31, x_63, x_64); -x_71 = lean_string_append(x_69, x_70); -lean_dec(x_70); -x_72 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__5; -x_73 = lean_string_append(x_71, x_72); -lean_ctor_set_tag(x_34, 3); -lean_ctor_set(x_34, 0, x_73); -x_74 = l_Lean_MessageData_ofFormat(x_34); -lean_inc(x_10); -x_75 = l_Lean_logWarning___at_Lean_Elab_Term_mkConst___spec__4(x_74, x_6, x_7, x_8, x_9, x_10, x_11, x_56); -x_76 = lean_ctor_get(x_75, 0); -lean_inc(x_76); -x_77 = lean_ctor_get(x_75, 1); -lean_inc(x_77); -lean_dec(x_75); -x_78 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___lambda__5(x_1, x_3, x_5, x_28, x_2, x_4, x_76, x_6, x_7, x_8, x_9, x_10, x_11, x_77); -lean_dec(x_76); -return x_78; -} -} -else -{ -lean_object* x_79; lean_object* x_80; uint8_t x_81; -x_79 = lean_ctor_get(x_34, 0); -lean_inc(x_79); -lean_dec(x_34); -x_80 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___closed__1; -x_81 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_20, x_80); -lean_dec(x_20); -if (x_81 == 0) -{ -lean_object* x_82; lean_object* x_83; -lean_dec(x_79); -lean_dec(x_31); -x_82 = lean_box(0); -x_83 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___lambda__5(x_1, x_3, x_5, x_28, x_2, x_4, x_82, x_6, x_7, x_8, x_9, x_10, x_11, x_56); -return x_83; -} -else -{ -uint8_t x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; -x_84 = 1; -x_85 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___closed__1; -x_86 = l_Lean_Name_toString(x_79, x_84, x_85); -x_87 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__1; -x_88 = lean_string_append(x_87, x_86); -lean_dec(x_86); -x_89 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__3; -x_90 = lean_string_append(x_88, x_89); -x_91 = l_Lean_Name_toString(x_31, x_84, x_85); -x_92 = lean_string_append(x_90, x_91); -lean_dec(x_91); -x_93 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__5; -x_94 = lean_string_append(x_92, x_93); -x_95 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_95, 0, x_94); -x_96 = l_Lean_MessageData_ofFormat(x_95); -lean_inc(x_10); -x_97 = l_Lean_logWarning___at_Lean_Elab_Term_mkConst___spec__4(x_96, x_6, x_7, x_8, x_9, x_10, x_11, x_56); -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_Structure_0__Lean_Elab_Command_withParents_go___rarg___lambda__5(x_1, x_3, x_5, x_28, x_2, x_4, x_98, x_6, x_7, x_8, x_9, x_10, x_11, x_99); -lean_dec(x_98); -return x_100; -} -} -} -} -else -{ -uint8_t x_101; -lean_dec(x_28); -lean_dec(x_10); -lean_dec(x_20); -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); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_101 = !lean_is_exclusive(x_30); -if (x_101 == 0) -{ -return x_30; -} -else -{ -lean_object* x_102; lean_object* x_103; lean_object* x_104; -x_102 = lean_ctor_get(x_30, 0); -x_103 = lean_ctor_get(x_30, 1); -lean_inc(x_103); -lean_inc(x_102); -lean_dec(x_30); -x_104 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_104, 0, x_102); -lean_ctor_set(x_104, 1, x_103); -return x_104; -} -} -} -else -{ -uint8_t x_105; -lean_dec(x_10); -lean_dec(x_20); -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); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_105 = !lean_is_exclusive(x_27); -if (x_105 == 0) -{ -return x_27; -} -else -{ -lean_object* x_106; lean_object* x_107; lean_object* x_108; -x_106 = lean_ctor_get(x_27, 0); -x_107 = lean_ctor_get(x_27, 1); -lean_inc(x_107); -lean_inc(x_106); -lean_dec(x_27); -x_108 = lean_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_109; -lean_dec(x_10); -lean_dec(x_20); -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); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_109 = !lean_is_exclusive(x_24); -if (x_109 == 0) -{ -return x_24; -} -else -{ -lean_object* x_110; lean_object* x_111; lean_object* x_112; -x_110 = lean_ctor_get(x_24, 0); -x_111 = lean_ctor_get(x_24, 1); -lean_inc(x_111); -lean_inc(x_110); -lean_dec(x_24); -x_112 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_112, 0, x_110); -lean_ctor_set(x_112, 1, x_111); -return x_112; -} -} -} -else -{ -lean_object* x_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; uint8_t x_126; lean_object* x_127; lean_object* x_128; uint8_t x_129; lean_object* x_130; -x_113 = lean_ctor_get(x_10, 0); -x_114 = lean_ctor_get(x_10, 1); -x_115 = lean_ctor_get(x_10, 2); -x_116 = lean_ctor_get(x_10, 3); -x_117 = lean_ctor_get(x_10, 4); -x_118 = lean_ctor_get(x_10, 5); -x_119 = lean_ctor_get(x_10, 6); -x_120 = lean_ctor_get(x_10, 7); -x_121 = lean_ctor_get(x_10, 8); -x_122 = lean_ctor_get(x_10, 9); -x_123 = lean_ctor_get(x_10, 10); -x_124 = lean_ctor_get_uint8(x_10, sizeof(void*)*12); -x_125 = lean_ctor_get(x_10, 11); -x_126 = lean_ctor_get_uint8(x_10, sizeof(void*)*12 + 1); -lean_inc(x_125); -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_inc(x_115); -lean_inc(x_114); -lean_inc(x_113); -lean_dec(x_10); -x_127 = l_Lean_replaceRef(x_17, x_118); -lean_dec(x_118); -lean_dec(x_17); -lean_inc(x_115); -x_128 = lean_alloc_ctor(0, 12, 2); -lean_ctor_set(x_128, 0, x_113); -lean_ctor_set(x_128, 1, x_114); -lean_ctor_set(x_128, 2, x_115); -lean_ctor_set(x_128, 3, x_116); -lean_ctor_set(x_128, 4, x_117); -lean_ctor_set(x_128, 5, x_127); -lean_ctor_set(x_128, 6, x_119); -lean_ctor_set(x_128, 7, x_120); -lean_ctor_set(x_128, 8, x_121); -lean_ctor_set(x_128, 9, x_122); -lean_ctor_set(x_128, 10, x_123); -lean_ctor_set(x_128, 11, x_125); -lean_ctor_set_uint8(x_128, sizeof(void*)*12, x_124); -lean_ctor_set_uint8(x_128, sizeof(void*)*12 + 1, x_126); -x_129 = 1; -lean_inc(x_11); -lean_inc(x_128); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -x_130 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_withSynthesizeImp___rarg(x_18, x_129, x_6, x_7, x_8, x_9, x_128, x_11, x_12); -if (lean_obj_tag(x_130) == 0) -{ -lean_object* x_131; lean_object* x_132; lean_object* x_133; -x_131 = lean_ctor_get(x_130, 0); -lean_inc(x_131); -x_132 = lean_ctor_get(x_130, 1); -lean_inc(x_132); -lean_dec(x_130); -lean_inc(x_11); -lean_inc(x_128); -lean_inc(x_9); -lean_inc(x_8); -x_133 = lean_whnf(x_131, x_8, x_9, x_128, x_11, x_132); -if (lean_obj_tag(x_133) == 0) -{ -lean_object* x_134; lean_object* x_135; lean_object* x_136; -x_134 = lean_ctor_get(x_133, 0); -lean_inc(x_134); -x_135 = lean_ctor_get(x_133, 1); -lean_inc(x_135); -lean_dec(x_133); -x_136 = l_Lean_Meta_getStructureName(x_134, x_8, x_9, x_128, x_11, x_135); -if (lean_obj_tag(x_136) == 0) -{ -lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; -x_137 = lean_ctor_get(x_136, 0); -lean_inc(x_137); -x_138 = lean_ctor_get(x_136, 1); -lean_inc(x_138); -lean_dec(x_136); -lean_inc(x_137); -x_139 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f(x_4, x_137, x_128, x_11, x_138); -x_140 = lean_ctor_get(x_139, 0); -lean_inc(x_140); -if (lean_obj_tag(x_140) == 0) -{ -lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; uint8_t x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; uint8_t x_150; lean_object* x_151; -lean_dec(x_115); -x_141 = lean_ctor_get(x_139, 1); -lean_inc(x_141); -lean_dec(x_139); -x_142 = lean_st_ref_get(x_11, x_141); -x_143 = lean_ctor_get(x_142, 0); -lean_inc(x_143); -x_144 = lean_ctor_get(x_142, 1); -lean_inc(x_144); -lean_dec(x_142); -x_145 = lean_ctor_get(x_143, 0); -lean_inc(x_145); -lean_dec(x_143); -x_146 = 1; -lean_inc(x_137); -x_147 = l_Lean_getStructureFieldsFlattened(x_145, x_137, x_146); -lean_inc(x_147); -lean_inc(x_4); -x_148 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___lambda__1___boxed), 3, 2); -lean_closure_set(x_148, 0, x_4); -lean_closure_set(x_148, 1, x_147); -lean_inc(x_137); -x_149 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkToParentName(x_137, x_148); -x_150 = lean_ctor_get_uint8(x_1, sizeof(void*)*11); -lean_inc(x_137); -lean_inc(x_149); -x_151 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___lambda__3), 16, 8); -lean_closure_set(x_151, 0, x_1); -lean_closure_set(x_151, 1, x_149); -lean_closure_set(x_151, 2, x_4); -lean_closure_set(x_151, 3, x_3); -lean_closure_set(x_151, 4, x_2); -lean_closure_set(x_151, 5, x_5); -lean_closure_set(x_151, 6, x_137); -lean_closure_set(x_151, 7, x_147); -if (x_150 == 0) -{ -uint8_t x_152; uint8_t x_153; lean_object* x_154; -lean_dec(x_145); -lean_dec(x_137); -x_152 = 0; -x_153 = 0; -x_154 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__1___rarg(x_149, x_152, x_134, x_151, x_153, x_6, x_7, x_8, x_9, x_128, x_11, x_144); -return x_154; -} -else -{ -uint8_t x_155; -x_155 = lean_is_class(x_145, x_137); -if (x_155 == 0) -{ -uint8_t x_156; uint8_t x_157; lean_object* x_158; -x_156 = 0; -x_157 = 0; -x_158 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__1___rarg(x_149, x_156, x_134, x_151, x_157, x_6, x_7, x_8, x_9, x_128, x_11, x_144); -return x_158; -} -else -{ -uint8_t x_159; uint8_t x_160; lean_object* x_161; -x_159 = 3; -x_160 = 0; -x_161 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__1___rarg(x_149, x_159, x_134, x_151, x_160, x_6, x_7, x_8, x_9, x_128, x_11, x_144); -return x_161; -} -} -} -else -{ -lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; uint8_t x_166; -x_162 = lean_ctor_get(x_139, 1); -lean_inc(x_162); -lean_dec(x_139); -x_163 = lean_ctor_get(x_140, 0); -lean_inc(x_163); -if (lean_is_exclusive(x_140)) { - lean_ctor_release(x_140, 0); - x_164 = x_140; -} else { - lean_dec_ref(x_140); - x_164 = lean_box(0); -} -x_165 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___closed__1; -x_166 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_115, x_165); -lean_dec(x_115); -if (x_166 == 0) -{ -lean_object* x_167; lean_object* x_168; -lean_dec(x_164); -lean_dec(x_163); -lean_dec(x_137); -x_167 = lean_box(0); -x_168 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___lambda__5(x_1, x_3, x_5, x_134, x_2, x_4, x_167, x_6, x_7, x_8, x_9, x_128, x_11, x_162); -return x_168; -} -else -{ -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; 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; -x_169 = 1; -x_170 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___closed__1; -x_171 = l_Lean_Name_toString(x_163, x_169, x_170); -x_172 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__1; -x_173 = lean_string_append(x_172, x_171); -lean_dec(x_171); -x_174 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__3; -x_175 = lean_string_append(x_173, x_174); -x_176 = l_Lean_Name_toString(x_137, x_169, x_170); -x_177 = lean_string_append(x_175, x_176); -lean_dec(x_176); -x_178 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__5; -x_179 = lean_string_append(x_177, x_178); -if (lean_is_scalar(x_164)) { - x_180 = lean_alloc_ctor(3, 1, 0); -} else { - x_180 = x_164; - lean_ctor_set_tag(x_180, 3); -} -lean_ctor_set(x_180, 0, x_179); -x_181 = l_Lean_MessageData_ofFormat(x_180); -lean_inc(x_128); -x_182 = l_Lean_logWarning___at_Lean_Elab_Term_mkConst___spec__4(x_181, x_6, x_7, x_8, x_9, x_128, x_11, x_162); -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_Structure_0__Lean_Elab_Command_withParents_go___rarg___lambda__5(x_1, x_3, x_5, x_134, x_2, x_4, x_183, x_6, x_7, x_8, x_9, x_128, x_11, x_184); -lean_dec(x_183); -return x_185; -} -} -} -else -{ -lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; -lean_dec(x_134); -lean_dec(x_128); -lean_dec(x_115); -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); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_186 = lean_ctor_get(x_136, 0); -lean_inc(x_186); -x_187 = lean_ctor_get(x_136, 1); -lean_inc(x_187); -if (lean_is_exclusive(x_136)) { - lean_ctor_release(x_136, 0); - lean_ctor_release(x_136, 1); - x_188 = x_136; -} else { - lean_dec_ref(x_136); - x_188 = lean_box(0); -} -if (lean_is_scalar(x_188)) { - x_189 = lean_alloc_ctor(1, 2, 0); -} else { - x_189 = x_188; -} -lean_ctor_set(x_189, 0, x_186); -lean_ctor_set(x_189, 1, x_187); -return x_189; -} -} -else -{ -lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; -lean_dec(x_128); -lean_dec(x_115); -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); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_190 = lean_ctor_get(x_133, 0); -lean_inc(x_190); -x_191 = lean_ctor_get(x_133, 1); -lean_inc(x_191); -if (lean_is_exclusive(x_133)) { - lean_ctor_release(x_133, 0); - lean_ctor_release(x_133, 1); - x_192 = x_133; -} else { - lean_dec_ref(x_133); - 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; -} -} -else -{ -lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; -lean_dec(x_128); -lean_dec(x_115); -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); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_194 = lean_ctor_get(x_130, 0); -lean_inc(x_194); -x_195 = lean_ctor_get(x_130, 1); -lean_inc(x_195); -if (lean_is_exclusive(x_130)) { - lean_ctor_release(x_130, 0); - lean_ctor_release(x_130, 1); - x_196 = x_130; -} else { - lean_dec_ref(x_130); - x_196 = lean_box(0); -} -if (lean_is_scalar(x_196)) { - x_197 = lean_alloc_ctor(1, 2, 0); -} else { - x_197 = x_196; -} -lean_ctor_set(x_197, 0, x_194); -lean_ctor_set(x_197, 1, x_195); -return x_197; -} -} -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg), 12, 0); -return x_2; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -uint8_t x_4; lean_object* x_5; -x_4 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___lambda__1(x_1, x_2, x_3); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_5 = lean_box(x_4); -return x_5; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_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, 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_Structure_0__Lean_Elab_Command_withParents_go___rarg___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_1); -return x_13; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { -_start: -{ -lean_object* x_14; -x_14 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_1); -return x_14; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { -_start: -{ -lean_object* x_15; -x_15 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -lean_dec(x_7); -return x_15; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents___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; -x_10 = lean_unsigned_to_nat(0u); -x_11 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; -x_12 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg(x_1, x_2, x_10, x_11, x_11, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_12; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents___rarg), 9, 0); -return x_2; -} -} -LEAN_EXPORT uint8_t l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabFieldTypeValue___lambda__1(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; uint8_t x_4; -x_3 = lean_ctor_get(x_1, 3); -x_4 = lean_name_eq(x_3, x_2); -return x_4; -} -} -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabFieldTypeValue___lambda__2___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = lean_box(0); -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_Elab_Structure_0__Lean_Elab_Command_elabFieldTypeValue___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; -x_10 = lean_ctor_get(x_1, 6); -lean_inc(x_10); -if (lean_obj_tag(x_10) == 0) -{ -lean_object* x_11; -x_11 = lean_ctor_get(x_1, 7); -lean_inc(x_11); -lean_dec(x_1); -if (lean_obj_tag(x_11) == 0) -{ -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); -x_12 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabFieldTypeValue___lambda__2___closed__1; -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_12); -lean_ctor_set(x_13, 1, x_9); -return x_13; -} -else -{ -uint8_t x_14; -x_14 = !lean_is_exclusive(x_11); -if (x_14 == 0) -{ -lean_object* x_15; uint8_t x_16; uint8_t x_17; lean_object* x_18; -x_15 = lean_ctor_get(x_11, 0); -x_16 = 1; -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_18 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_16, x_17, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -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); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_3); -x_20 = l_Lean_Elab_Term_addAutoBoundImplicits(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_19); -if (lean_obj_tag(x_20) == 0) -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; -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_box(0); -x_24 = 1; -x_25 = lean_box(x_24); -x_26 = lean_box(x_24); -x_27 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTerm___boxed), 11, 4); -lean_closure_set(x_27, 0, x_15); -lean_closure_set(x_27, 1, x_23); -lean_closure_set(x_27, 2, x_25); -lean_closure_set(x_27, 3, x_26); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -x_28 = l_Lean_Elab_Term_withoutAutoBoundImplicit___rarg(x_27, x_3, x_4, x_5, x_6, x_7, x_8, x_22); -if (lean_obj_tag(x_28) == 0) -{ -lean_object* x_29; lean_object* x_30; uint8_t x_31; lean_object* x_32; -x_29 = lean_ctor_get(x_28, 0); -lean_inc(x_29); -x_30 = lean_ctor_get(x_28, 1); -lean_inc(x_30); -lean_dec(x_28); -x_31 = 1; -x_32 = l_Lean_Meta_mkLambdaFVars(x_21, x_29, x_17, x_24, x_17, x_31, 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); -if (lean_obj_tag(x_32) == 0) -{ -uint8_t x_33; -x_33 = !lean_is_exclusive(x_32); -if (x_33 == 0) -{ -lean_object* x_34; lean_object* x_35; -x_34 = lean_ctor_get(x_32, 0); -lean_ctor_set(x_11, 0, x_34); -x_35 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_35, 0, x_23); -lean_ctor_set(x_35, 1, x_11); -lean_ctor_set(x_32, 0, x_35); -return x_32; -} -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); -lean_ctor_set(x_11, 0, x_36); -x_38 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_38, 0, x_23); -lean_ctor_set(x_38, 1, x_11); -x_39 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_39, 0, x_38); -lean_ctor_set(x_39, 1, x_37); -return x_39; -} -} -else -{ -uint8_t x_40; -lean_free_object(x_11); -x_40 = !lean_is_exclusive(x_32); -if (x_40 == 0) -{ -return x_32; -} -else -{ -lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_ctor_get(x_32, 0); -x_42 = lean_ctor_get(x_32, 1); -lean_inc(x_42); -lean_inc(x_41); -lean_dec(x_32); -x_43 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_43, 0, x_41); -lean_ctor_set(x_43, 1, x_42); -return x_43; -} -} -} -else -{ -uint8_t x_44; -lean_dec(x_21); -lean_free_object(x_11); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -x_44 = !lean_is_exclusive(x_28); -if (x_44 == 0) -{ -return x_28; -} -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; -} -} -} -else -{ -uint8_t x_48; -lean_free_object(x_11); -lean_dec(x_15); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_48 = !lean_is_exclusive(x_20); -if (x_48 == 0) -{ -return x_20; -} -else -{ -lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_49 = lean_ctor_get(x_20, 0); -x_50 = lean_ctor_get(x_20, 1); -lean_inc(x_50); -lean_inc(x_49); -lean_dec(x_20); -x_51 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_51, 0, x_49); -lean_ctor_set(x_51, 1, x_50); -return x_51; -} -} -} -else -{ -uint8_t x_52; -lean_free_object(x_11); -lean_dec(x_15); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_52 = !lean_is_exclusive(x_18); -if (x_52 == 0) -{ -return x_18; -} -else -{ -lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_53 = lean_ctor_get(x_18, 0); -x_54 = lean_ctor_get(x_18, 1); -lean_inc(x_54); -lean_inc(x_53); -lean_dec(x_18); -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; uint8_t x_57; uint8_t x_58; lean_object* x_59; -x_56 = lean_ctor_get(x_11, 0); -lean_inc(x_56); -lean_dec(x_11); -x_57 = 1; -x_58 = 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_59 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_57, x_58, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_59) == 0) -{ -lean_object* x_60; lean_object* x_61; -x_60 = lean_ctor_get(x_59, 1); -lean_inc(x_60); -lean_dec(x_59); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_3); -x_61 = l_Lean_Elab_Term_addAutoBoundImplicits(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_60); -if (lean_obj_tag(x_61) == 0) -{ -lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_62 = lean_ctor_get(x_61, 0); -lean_inc(x_62); -x_63 = lean_ctor_get(x_61, 1); -lean_inc(x_63); -lean_dec(x_61); -x_64 = lean_box(0); -x_65 = 1; -x_66 = lean_box(x_65); -x_67 = lean_box(x_65); -x_68 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTerm___boxed), 11, 4); -lean_closure_set(x_68, 0, x_56); -lean_closure_set(x_68, 1, x_64); -lean_closure_set(x_68, 2, x_66); -lean_closure_set(x_68, 3, x_67); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -x_69 = l_Lean_Elab_Term_withoutAutoBoundImplicit___rarg(x_68, x_3, x_4, x_5, x_6, x_7, x_8, x_63); -if (lean_obj_tag(x_69) == 0) -{ -lean_object* x_70; lean_object* x_71; uint8_t x_72; lean_object* x_73; -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 = 1; -x_73 = l_Lean_Meta_mkLambdaFVars(x_62, x_70, x_58, x_65, x_58, x_72, x_5, x_6, x_7, x_8, x_71); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -if (lean_obj_tag(x_73) == 0) -{ -lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; -x_74 = lean_ctor_get(x_73, 0); -lean_inc(x_74); -x_75 = lean_ctor_get(x_73, 1); -lean_inc(x_75); -if (lean_is_exclusive(x_73)) { - lean_ctor_release(x_73, 0); - lean_ctor_release(x_73, 1); - x_76 = x_73; -} else { - lean_dec_ref(x_73); - x_76 = lean_box(0); -} -x_77 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_77, 0, x_74); -x_78 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_78, 0, x_64); -lean_ctor_set(x_78, 1, x_77); -if (lean_is_scalar(x_76)) { - x_79 = lean_alloc_ctor(0, 2, 0); -} else { - x_79 = x_76; -} -lean_ctor_set(x_79, 0, x_78); -lean_ctor_set(x_79, 1, x_75); -return x_79; -} -else -{ -lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; -x_80 = lean_ctor_get(x_73, 0); -lean_inc(x_80); -x_81 = lean_ctor_get(x_73, 1); -lean_inc(x_81); -if (lean_is_exclusive(x_73)) { - lean_ctor_release(x_73, 0); - lean_ctor_release(x_73, 1); - x_82 = x_73; -} else { - lean_dec_ref(x_73); - x_82 = lean_box(0); -} -if (lean_is_scalar(x_82)) { - x_83 = lean_alloc_ctor(1, 2, 0); -} else { - x_83 = x_82; -} -lean_ctor_set(x_83, 0, x_80); -lean_ctor_set(x_83, 1, x_81); -return x_83; -} -} -else -{ -lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; -lean_dec(x_62); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -x_84 = lean_ctor_get(x_69, 0); -lean_inc(x_84); -x_85 = lean_ctor_get(x_69, 1); -lean_inc(x_85); -if (lean_is_exclusive(x_69)) { - lean_ctor_release(x_69, 0); - lean_ctor_release(x_69, 1); - x_86 = x_69; -} else { - lean_dec_ref(x_69); - x_86 = lean_box(0); -} -if (lean_is_scalar(x_86)) { - x_87 = lean_alloc_ctor(1, 2, 0); -} else { - x_87 = x_86; -} -lean_ctor_set(x_87, 0, x_84); -lean_ctor_set(x_87, 1, x_85); -return x_87; -} -} -else -{ -lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; -lean_dec(x_56); -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_88 = lean_ctor_get(x_61, 0); -lean_inc(x_88); -x_89 = lean_ctor_get(x_61, 1); -lean_inc(x_89); -if (lean_is_exclusive(x_61)) { - lean_ctor_release(x_61, 0); - lean_ctor_release(x_61, 1); - x_90 = x_61; -} else { - lean_dec_ref(x_61); - x_90 = lean_box(0); -} -if (lean_is_scalar(x_90)) { - x_91 = lean_alloc_ctor(1, 2, 0); -} else { - x_91 = x_90; -} -lean_ctor_set(x_91, 0, x_88); -lean_ctor_set(x_91, 1, x_89); -return x_91; -} -} -else -{ -lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; -lean_dec(x_56); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_92 = lean_ctor_get(x_59, 0); -lean_inc(x_92); -x_93 = lean_ctor_get(x_59, 1); -lean_inc(x_93); -if (lean_is_exclusive(x_59)) { - lean_ctor_release(x_59, 0); - lean_ctor_release(x_59, 1); - x_94 = x_59; -} else { - lean_dec_ref(x_59); - x_94 = lean_box(0); -} -if (lean_is_scalar(x_94)) { - x_95 = lean_alloc_ctor(1, 2, 0); -} else { - x_95 = x_94; -} -lean_ctor_set(x_95, 0, x_92); -lean_ctor_set(x_95, 1, x_93); -return x_95; -} -} -} -} -else -{ -uint8_t x_96; -x_96 = !lean_is_exclusive(x_10); -if (x_96 == 0) -{ -lean_object* x_97; lean_object* x_98; -x_97 = 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_98 = l_Lean_Elab_Term_elabType(x_97, x_3, x_4, x_5, 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; uint8_t x_102; lean_object* x_103; -x_99 = lean_ctor_get(x_98, 0); -lean_inc(x_99); -x_100 = lean_ctor_get(x_98, 1); -lean_inc(x_100); -lean_dec(x_98); -x_101 = 1; -x_102 = 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_103 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_101, x_102, x_3, x_4, x_5, x_6, x_7, x_8, x_100); -if (lean_obj_tag(x_103) == 0) -{ -lean_object* x_104; lean_object* x_105; -x_104 = lean_ctor_get(x_103, 1); -lean_inc(x_104); -lean_dec(x_103); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_3); -x_105 = l_Lean_Elab_Term_addAutoBoundImplicits(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_104); -if (lean_obj_tag(x_105) == 0) -{ -lean_object* x_106; -x_106 = lean_ctor_get(x_1, 7); -lean_inc(x_106); -lean_dec(x_1); -if (lean_obj_tag(x_106) == 0) -{ -lean_object* x_107; lean_object* x_108; uint8_t x_109; uint8_t x_110; lean_object* x_111; -lean_dec(x_4); -lean_dec(x_3); -x_107 = lean_ctor_get(x_105, 0); -lean_inc(x_107); -x_108 = lean_ctor_get(x_105, 1); -lean_inc(x_108); -lean_dec(x_105); -x_109 = 1; -x_110 = 1; -x_111 = l_Lean_Meta_mkForallFVars(x_107, x_99, x_102, x_109, x_110, x_5, x_6, x_7, x_8, x_108); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -if (lean_obj_tag(x_111) == 0) -{ -uint8_t x_112; -x_112 = !lean_is_exclusive(x_111); -if (x_112 == 0) -{ -lean_object* x_113; lean_object* x_114; lean_object* x_115; -x_113 = lean_ctor_get(x_111, 0); -lean_ctor_set(x_10, 0, x_113); -x_114 = lean_box(0); -x_115 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_115, 0, x_10); -lean_ctor_set(x_115, 1, x_114); -lean_ctor_set(x_111, 0, x_115); -return x_111; -} -else -{ -lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; -x_116 = lean_ctor_get(x_111, 0); -x_117 = lean_ctor_get(x_111, 1); -lean_inc(x_117); -lean_inc(x_116); -lean_dec(x_111); -lean_ctor_set(x_10, 0, x_116); -x_118 = lean_box(0); -x_119 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_119, 0, x_10); -lean_ctor_set(x_119, 1, x_118); -x_120 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_120, 0, x_119); -lean_ctor_set(x_120, 1, x_117); -return x_120; -} -} -else -{ -uint8_t x_121; -lean_free_object(x_10); -x_121 = !lean_is_exclusive(x_111); -if (x_121 == 0) -{ -return x_111; -} -else -{ -lean_object* x_122; lean_object* x_123; lean_object* x_124; -x_122 = lean_ctor_get(x_111, 0); -x_123 = lean_ctor_get(x_111, 1); -lean_inc(x_123); -lean_inc(x_122); -lean_dec(x_111); -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 -{ -lean_object* x_125; lean_object* x_126; uint8_t x_127; -x_125 = lean_ctor_get(x_105, 0); -lean_inc(x_125); -x_126 = lean_ctor_get(x_105, 1); -lean_inc(x_126); -lean_dec(x_105); -x_127 = !lean_is_exclusive(x_106); -if (x_127 == 0) -{ -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; -x_128 = lean_ctor_get(x_106, 0); -lean_inc(x_99); -lean_ctor_set(x_106, 0, x_99); -x_129 = lean_box(0); -x_130 = 1; -x_131 = lean_box(x_130); -x_132 = lean_box(x_130); -x_133 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTermEnsuringType___boxed), 12, 5); -lean_closure_set(x_133, 0, x_128); -lean_closure_set(x_133, 1, x_106); -lean_closure_set(x_133, 2, x_131); -lean_closure_set(x_133, 3, x_132); -lean_closure_set(x_133, 4, x_129); -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_134 = l_Lean_Elab_Term_withoutAutoBoundImplicit___rarg(x_133, x_3, x_4, x_5, x_6, x_7, x_8, x_126); -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_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -x_137 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_101, x_102, x_3, x_4, x_5, x_6, x_7, x_8, x_136); -if (lean_obj_tag(x_137) == 0) -{ -lean_object* x_138; uint8_t x_139; lean_object* x_140; -x_138 = lean_ctor_get(x_137, 1); -lean_inc(x_138); -lean_dec(x_137); -x_139 = 1; -lean_inc(x_125); -x_140 = l_Lean_Meta_mkForallFVars(x_125, x_99, x_102, x_130, x_139, x_5, x_6, x_7, x_8, x_138); -if (lean_obj_tag(x_140) == 0) -{ -lean_object* x_141; lean_object* x_142; lean_object* x_143; -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 = l_Lean_Meta_mkLambdaFVars(x_125, x_135, x_102, x_130, x_102, x_139, x_5, x_6, x_7, x_8, x_142); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -if (lean_obj_tag(x_143) == 0) -{ -uint8_t x_144; -x_144 = !lean_is_exclusive(x_143); -if (x_144 == 0) -{ -lean_object* x_145; lean_object* x_146; lean_object* x_147; -x_145 = lean_ctor_get(x_143, 0); -lean_ctor_set(x_10, 0, x_141); -x_146 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_146, 0, x_145); -x_147 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_147, 0, x_10); -lean_ctor_set(x_147, 1, x_146); -lean_ctor_set(x_143, 0, x_147); -return x_143; -} -else -{ -lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; -x_148 = lean_ctor_get(x_143, 0); -x_149 = lean_ctor_get(x_143, 1); -lean_inc(x_149); -lean_inc(x_148); -lean_dec(x_143); -lean_ctor_set(x_10, 0, x_141); -x_150 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_150, 0, x_148); -x_151 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_151, 0, x_10); -lean_ctor_set(x_151, 1, x_150); -x_152 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_152, 0, x_151); -lean_ctor_set(x_152, 1, x_149); -return x_152; -} -} -else -{ -uint8_t x_153; -lean_dec(x_141); -lean_free_object(x_10); -x_153 = !lean_is_exclusive(x_143); -if (x_153 == 0) -{ -return x_143; -} -else -{ -lean_object* x_154; lean_object* x_155; lean_object* x_156; -x_154 = lean_ctor_get(x_143, 0); -x_155 = lean_ctor_get(x_143, 1); -lean_inc(x_155); -lean_inc(x_154); -lean_dec(x_143); -x_156 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_156, 0, x_154); -lean_ctor_set(x_156, 1, x_155); -return x_156; -} -} -} -else -{ -uint8_t x_157; -lean_dec(x_135); -lean_dec(x_125); -lean_free_object(x_10); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -x_157 = !lean_is_exclusive(x_140); -if (x_157 == 0) -{ -return x_140; -} -else -{ -lean_object* x_158; lean_object* x_159; lean_object* x_160; -x_158 = lean_ctor_get(x_140, 0); -x_159 = lean_ctor_get(x_140, 1); -lean_inc(x_159); -lean_inc(x_158); -lean_dec(x_140); -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; -} -} -} -else -{ -uint8_t x_161; -lean_dec(x_135); -lean_dec(x_125); -lean_dec(x_99); -lean_free_object(x_10); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -x_161 = !lean_is_exclusive(x_137); -if (x_161 == 0) -{ -return x_137; -} -else -{ -lean_object* x_162; lean_object* x_163; lean_object* x_164; -x_162 = lean_ctor_get(x_137, 0); -x_163 = lean_ctor_get(x_137, 1); -lean_inc(x_163); -lean_inc(x_162); -lean_dec(x_137); -x_164 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_164, 0, x_162); -lean_ctor_set(x_164, 1, x_163); -return x_164; -} -} -} -else -{ -uint8_t x_165; -lean_dec(x_125); -lean_dec(x_99); -lean_free_object(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); -x_165 = !lean_is_exclusive(x_134); -if (x_165 == 0) -{ -return x_134; -} -else -{ -lean_object* x_166; lean_object* x_167; lean_object* x_168; -x_166 = lean_ctor_get(x_134, 0); -x_167 = lean_ctor_get(x_134, 1); -lean_inc(x_167); -lean_inc(x_166); -lean_dec(x_134); -x_168 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_168, 0, x_166); -lean_ctor_set(x_168, 1, x_167); -return x_168; -} -} -} -else -{ -lean_object* x_169; lean_object* x_170; lean_object* x_171; uint8_t x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; -x_169 = lean_ctor_get(x_106, 0); -lean_inc(x_169); -lean_dec(x_106); -lean_inc(x_99); -x_170 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_170, 0, x_99); -x_171 = lean_box(0); -x_172 = 1; -x_173 = lean_box(x_172); -x_174 = lean_box(x_172); -x_175 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTermEnsuringType___boxed), 12, 5); -lean_closure_set(x_175, 0, x_169); -lean_closure_set(x_175, 1, x_170); -lean_closure_set(x_175, 2, x_173); -lean_closure_set(x_175, 3, x_174); -lean_closure_set(x_175, 4, x_171); -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_176 = l_Lean_Elab_Term_withoutAutoBoundImplicit___rarg(x_175, x_3, x_4, x_5, x_6, x_7, x_8, x_126); -if (lean_obj_tag(x_176) == 0) -{ -lean_object* x_177; lean_object* x_178; lean_object* x_179; -x_177 = lean_ctor_get(x_176, 0); -lean_inc(x_177); -x_178 = lean_ctor_get(x_176, 1); -lean_inc(x_178); -lean_dec(x_176); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -x_179 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_101, x_102, x_3, x_4, x_5, x_6, x_7, x_8, x_178); -if (lean_obj_tag(x_179) == 0) -{ -lean_object* x_180; uint8_t x_181; lean_object* x_182; -x_180 = lean_ctor_get(x_179, 1); -lean_inc(x_180); -lean_dec(x_179); -x_181 = 1; -lean_inc(x_125); -x_182 = l_Lean_Meta_mkForallFVars(x_125, x_99, x_102, x_172, x_181, x_5, x_6, x_7, x_8, x_180); -if (lean_obj_tag(x_182) == 0) -{ -lean_object* x_183; lean_object* x_184; lean_object* x_185; -x_183 = lean_ctor_get(x_182, 0); -lean_inc(x_183); -x_184 = lean_ctor_get(x_182, 1); -lean_inc(x_184); -lean_dec(x_182); -x_185 = l_Lean_Meta_mkLambdaFVars(x_125, x_177, x_102, x_172, x_102, x_181, x_5, x_6, x_7, x_8, x_184); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -if (lean_obj_tag(x_185) == 0) -{ -lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; -x_186 = lean_ctor_get(x_185, 0); -lean_inc(x_186); -x_187 = lean_ctor_get(x_185, 1); -lean_inc(x_187); -if (lean_is_exclusive(x_185)) { - lean_ctor_release(x_185, 0); - lean_ctor_release(x_185, 1); - x_188 = x_185; -} else { - lean_dec_ref(x_185); - x_188 = lean_box(0); -} -lean_ctor_set(x_10, 0, x_183); -x_189 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_189, 0, x_186); -x_190 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_190, 0, x_10); -lean_ctor_set(x_190, 1, x_189); -if (lean_is_scalar(x_188)) { - x_191 = lean_alloc_ctor(0, 2, 0); -} else { - x_191 = x_188; -} -lean_ctor_set(x_191, 0, x_190); -lean_ctor_set(x_191, 1, x_187); -return x_191; -} -else -{ -lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; -lean_dec(x_183); -lean_free_object(x_10); -x_192 = lean_ctor_get(x_185, 0); -lean_inc(x_192); -x_193 = lean_ctor_get(x_185, 1); -lean_inc(x_193); -if (lean_is_exclusive(x_185)) { - lean_ctor_release(x_185, 0); - lean_ctor_release(x_185, 1); - x_194 = x_185; -} else { - lean_dec_ref(x_185); - x_194 = lean_box(0); -} -if (lean_is_scalar(x_194)) { - x_195 = lean_alloc_ctor(1, 2, 0); -} else { - x_195 = x_194; -} -lean_ctor_set(x_195, 0, x_192); -lean_ctor_set(x_195, 1, x_193); -return x_195; -} -} -else -{ -lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; -lean_dec(x_177); -lean_dec(x_125); -lean_free_object(x_10); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -x_196 = lean_ctor_get(x_182, 0); -lean_inc(x_196); -x_197 = lean_ctor_get(x_182, 1); -lean_inc(x_197); -if (lean_is_exclusive(x_182)) { - lean_ctor_release(x_182, 0); - lean_ctor_release(x_182, 1); - x_198 = x_182; -} else { - lean_dec_ref(x_182); - 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_177); -lean_dec(x_125); -lean_dec(x_99); -lean_free_object(x_10); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -x_200 = lean_ctor_get(x_179, 0); -lean_inc(x_200); -x_201 = lean_ctor_get(x_179, 1); -lean_inc(x_201); -if (lean_is_exclusive(x_179)) { - lean_ctor_release(x_179, 0); - lean_ctor_release(x_179, 1); - x_202 = x_179; -} else { - lean_dec_ref(x_179); - 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; lean_object* x_206; lean_object* x_207; -lean_dec(x_125); -lean_dec(x_99); -lean_free_object(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); -x_204 = lean_ctor_get(x_176, 0); -lean_inc(x_204); -x_205 = lean_ctor_get(x_176, 1); -lean_inc(x_205); -if (lean_is_exclusive(x_176)) { - lean_ctor_release(x_176, 0); - lean_ctor_release(x_176, 1); - x_206 = x_176; -} else { - lean_dec_ref(x_176); - 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; -} -} -} -} -else -{ -uint8_t x_208; -lean_dec(x_99); -lean_free_object(x_10); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_208 = !lean_is_exclusive(x_105); -if (x_208 == 0) -{ -return x_105; -} -else -{ -lean_object* x_209; lean_object* x_210; lean_object* x_211; -x_209 = lean_ctor_get(x_105, 0); -x_210 = lean_ctor_get(x_105, 1); -lean_inc(x_210); -lean_inc(x_209); -lean_dec(x_105); -x_211 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_211, 0, x_209); -lean_ctor_set(x_211, 1, x_210); -return x_211; -} -} -} -else -{ -uint8_t x_212; -lean_dec(x_99); -lean_free_object(x_10); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_212 = !lean_is_exclusive(x_103); -if (x_212 == 0) -{ -return x_103; -} -else -{ -lean_object* x_213; lean_object* x_214; lean_object* x_215; -x_213 = lean_ctor_get(x_103, 0); -x_214 = lean_ctor_get(x_103, 1); -lean_inc(x_214); -lean_inc(x_213); -lean_dec(x_103); -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; -} -} -} -else -{ -uint8_t x_216; -lean_free_object(x_10); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_216 = !lean_is_exclusive(x_98); -if (x_216 == 0) -{ -return x_98; -} -else -{ -lean_object* x_217; lean_object* x_218; lean_object* x_219; -x_217 = lean_ctor_get(x_98, 0); -x_218 = lean_ctor_get(x_98, 1); -lean_inc(x_218); -lean_inc(x_217); -lean_dec(x_98); -x_219 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_219, 0, x_217); -lean_ctor_set(x_219, 1, x_218); -return x_219; -} -} -} -else -{ -lean_object* x_220; lean_object* x_221; -x_220 = lean_ctor_get(x_10, 0); -lean_inc(x_220); -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); -x_221 = l_Lean_Elab_Term_elabType(x_220, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_221) == 0) -{ -lean_object* x_222; lean_object* x_223; uint8_t x_224; uint8_t x_225; lean_object* x_226; -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 = 1; -x_225 = 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_226 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_224, x_225, x_3, x_4, x_5, x_6, x_7, x_8, x_223); -if (lean_obj_tag(x_226) == 0) -{ -lean_object* x_227; lean_object* x_228; -x_227 = lean_ctor_get(x_226, 1); -lean_inc(x_227); -lean_dec(x_226); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_3); -x_228 = l_Lean_Elab_Term_addAutoBoundImplicits(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_227); -if (lean_obj_tag(x_228) == 0) -{ -lean_object* x_229; -x_229 = lean_ctor_get(x_1, 7); -lean_inc(x_229); -lean_dec(x_1); -if (lean_obj_tag(x_229) == 0) -{ -lean_object* x_230; lean_object* x_231; uint8_t x_232; uint8_t x_233; lean_object* x_234; -lean_dec(x_4); -lean_dec(x_3); -x_230 = lean_ctor_get(x_228, 0); -lean_inc(x_230); -x_231 = lean_ctor_get(x_228, 1); -lean_inc(x_231); -lean_dec(x_228); -x_232 = 1; -x_233 = 1; -x_234 = l_Lean_Meta_mkForallFVars(x_230, x_222, x_225, x_232, x_233, x_5, x_6, x_7, x_8, x_231); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -if (lean_obj_tag(x_234) == 0) -{ -lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; -x_235 = lean_ctor_get(x_234, 0); -lean_inc(x_235); -x_236 = lean_ctor_get(x_234, 1); -lean_inc(x_236); -if (lean_is_exclusive(x_234)) { - lean_ctor_release(x_234, 0); - lean_ctor_release(x_234, 1); - x_237 = x_234; -} else { - lean_dec_ref(x_234); - x_237 = lean_box(0); -} -x_238 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_238, 0, x_235); -x_239 = lean_box(0); -x_240 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_240, 0, x_238); -lean_ctor_set(x_240, 1, x_239); -if (lean_is_scalar(x_237)) { - x_241 = lean_alloc_ctor(0, 2, 0); -} else { - x_241 = x_237; -} -lean_ctor_set(x_241, 0, x_240); -lean_ctor_set(x_241, 1, x_236); -return x_241; -} -else -{ -lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; -x_242 = lean_ctor_get(x_234, 0); -lean_inc(x_242); -x_243 = lean_ctor_get(x_234, 1); -lean_inc(x_243); -if (lean_is_exclusive(x_234)) { - lean_ctor_release(x_234, 0); - lean_ctor_release(x_234, 1); - x_244 = x_234; -} else { - lean_dec_ref(x_234); - x_244 = lean_box(0); -} -if (lean_is_scalar(x_244)) { - x_245 = lean_alloc_ctor(1, 2, 0); -} else { - x_245 = x_244; -} -lean_ctor_set(x_245, 0, x_242); -lean_ctor_set(x_245, 1, x_243); -return x_245; -} -} -else -{ -lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; uint8_t x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; -x_246 = lean_ctor_get(x_228, 0); -lean_inc(x_246); -x_247 = lean_ctor_get(x_228, 1); -lean_inc(x_247); -lean_dec(x_228); -x_248 = lean_ctor_get(x_229, 0); -lean_inc(x_248); -if (lean_is_exclusive(x_229)) { - lean_ctor_release(x_229, 0); - x_249 = x_229; -} else { - lean_dec_ref(x_229); - x_249 = lean_box(0); -} -lean_inc(x_222); -if (lean_is_scalar(x_249)) { - x_250 = lean_alloc_ctor(1, 1, 0); -} else { - x_250 = x_249; +lean_inc(x_222); +if (lean_is_scalar(x_249)) { + x_250 = lean_alloc_ctor(1, 1, 0); +} else { + x_250 = x_249; } lean_ctor_set(x_250, 0, x_222); x_251 = lean_box(0); @@ -17995,7 +15308,7 @@ lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_ lean_inc(x_1); x_9 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabFieldTypeValue___lambda__1___boxed), 2, 1); lean_closure_set(x_9, 0, x_1); -x_10 = lean_ctor_get(x_1, 5); +x_10 = lean_ctor_get(x_1, 6); lean_inc(x_10); x_11 = l_Lean_Syntax_getArgs(x_10); lean_dec(x_10); @@ -18815,161 +16128,178 @@ x_2 = lean_alloc_closure((void*)(l_Lean_throwErrorAt___at___private_Lean_Elab_St return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { _start: { -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; -x_17 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_17, 0, x_1); -x_18 = 0; -x_19 = lean_alloc_ctor(0, 4, 1); -lean_ctor_set(x_19, 0, x_2); -lean_ctor_set(x_19, 1, x_3); -lean_ctor_set(x_19, 2, x_9); -lean_ctor_set(x_19, 3, x_17); -lean_ctor_set_uint8(x_19, sizeof(void*)*4, x_18); -x_20 = lean_array_push(x_4, x_19); -x_21 = lean_unsigned_to_nat(1u); -x_22 = lean_nat_add(x_5, x_21); -x_23 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg(x_6, x_7, x_22, x_8, x_20, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -return x_23; +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; +x_18 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_18, 0, x_1); +x_19 = 0; +x_20 = lean_alloc_ctor(0, 5, 1); +lean_ctor_set(x_20, 0, x_2); +lean_ctor_set(x_20, 1, x_3); +lean_ctor_set(x_20, 2, x_4); +lean_ctor_set(x_20, 3, x_10); +lean_ctor_set(x_20, 4, x_18); +lean_ctor_set_uint8(x_20, sizeof(void*)*5, x_19); +x_21 = lean_array_push(x_5, x_20); +x_22 = lean_unsigned_to_nat(1u); +x_23 = lean_nat_add(x_6, x_22); +x_24 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg(x_7, x_8, x_23, x_9, x_21, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +return x_24; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_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, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_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, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { _start: { -uint8_t x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_17 = 0; -x_18 = lean_alloc_ctor(0, 4, 1); -lean_ctor_set(x_18, 0, x_1); -lean_ctor_set(x_18, 1, x_2); -lean_ctor_set(x_18, 2, x_9); -lean_ctor_set(x_18, 3, x_3); -lean_ctor_set_uint8(x_18, sizeof(void*)*4, x_17); -x_19 = lean_array_push(x_4, x_18); -x_20 = lean_unsigned_to_nat(1u); -x_21 = lean_nat_add(x_5, x_20); -x_22 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg(x_6, x_7, x_21, x_8, x_19, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -return x_22; +uint8_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_18 = 0; +x_19 = lean_alloc_ctor(0, 5, 1); +lean_ctor_set(x_19, 0, x_1); +lean_ctor_set(x_19, 1, x_2); +lean_ctor_set(x_19, 2, x_3); +lean_ctor_set(x_19, 3, x_10); +lean_ctor_set(x_19, 4, x_4); +lean_ctor_set_uint8(x_19, sizeof(void*)*5, x_18); +x_20 = lean_array_push(x_5, x_19); +x_21 = lean_unsigned_to_nat(1u); +x_22 = lean_nat_add(x_6, x_21); +x_23 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg(x_7, x_8, x_22, x_9, x_20, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +return x_23; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, 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_18; lean_object* x_19; -x_18 = lean_ctor_get(x_1, 2); +lean_object* x_21; +lean_inc(x_19); lean_inc(x_18); -lean_dec(x_1); +lean_inc(x_17); lean_inc(x_16); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -x_19 = lean_infer_type(x_18, x_13, x_14, x_15, x_16, x_17); -if (lean_obj_tag(x_19) == 0) +lean_inc(x_1); +x_21 = lean_infer_type(x_1, x_16, x_17, x_18, x_19, x_20); +if (lean_obj_tag(x_21) == 0) { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; lean_object* x_25; -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_19, 1); -lean_inc(x_21); -lean_dec(x_19); -x_22 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_22, 0, x_20); -x_23 = lean_box(0); -x_24 = 1; +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; lean_object* x_27; +x_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_ctor(1, 1, 0); +lean_ctor_set(x_24, 0, x_22); +x_25 = lean_box(0); +x_26 = 1; +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -x_25 = l_Lean_Elab_Term_elabTermEnsuringType(x_9, x_22, x_24, x_24, x_23, x_11, x_12, x_13, x_14, x_15, x_16, x_21); -if (lean_obj_tag(x_25) == 0) +x_27 = l_Lean_Elab_Term_elabTermEnsuringType(x_12, x_24, x_26, x_26, x_25, x_14, x_15, x_16, x_17, x_18, x_19, x_23); +if (lean_obj_tag(x_27) == 0) { -lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_26 = lean_ctor_get(x_25, 0); -lean_inc(x_26); -x_27 = lean_ctor_get(x_25, 1); -lean_inc(x_27); -lean_dec(x_25); -x_28 = lean_alloc_ctor(10, 1, 0); -lean_ctor_set(x_28, 0, x_2); -x_29 = l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Term_addDotCompletionInfo___spec__2(x_28, x_11, x_12, x_13, x_14, x_15, x_16, x_27); -x_30 = lean_ctor_get(x_29, 1); -lean_inc(x_30); -lean_dec(x_29); -x_31 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateFieldInfoVal(x_3, x_4, x_26); -x_32 = lean_unsigned_to_nat(1u); -x_33 = lean_nat_add(x_5, x_32); -x_34 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg(x_6, x_7, x_33, x_8, x_31, x_11, x_12, x_13, x_14, x_15, x_16, x_30); -return x_34; +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_28 = lean_ctor_get(x_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_alloc_ctor(10, 1, 0); +lean_ctor_set(x_30, 0, x_2); +x_31 = l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Term_addDotCompletionInfo___spec__2(x_30, x_14, x_15, x_16, x_17, x_18, x_19, x_29); +x_32 = lean_ctor_get(x_31, 1); +lean_inc(x_32); +lean_dec(x_31); +x_33 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_33, 0, x_28); +x_34 = lean_alloc_ctor(0, 5, 1); +lean_ctor_set(x_34, 0, x_3); +lean_ctor_set(x_34, 1, x_4); +lean_ctor_set(x_34, 2, x_5); +lean_ctor_set(x_34, 3, x_1); +lean_ctor_set(x_34, 4, x_33); +lean_ctor_set_uint8(x_34, sizeof(void*)*5, x_6); +x_35 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_replaceFieldInfo(x_7, x_34); +x_36 = lean_unsigned_to_nat(1u); +x_37 = lean_nat_add(x_8, x_36); +x_38 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg(x_9, x_10, x_37, x_11, x_35, x_14, x_15, x_16, x_17, x_18, x_19, x_32); +return x_38; } else { -uint8_t x_35; +uint8_t x_39; +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); lean_dec(x_11); -lean_dec(x_8); +lean_dec(x_10); +lean_dec(x_9); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_35 = !lean_is_exclusive(x_25); -if (x_35 == 0) +lean_dec(x_1); +x_39 = !lean_is_exclusive(x_27); +if (x_39 == 0) { -return x_25; +return x_27; } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_25, 0); -x_37 = lean_ctor_get(x_25, 1); -lean_inc(x_37); -lean_inc(x_36); -lean_dec(x_25); -x_38 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -return x_38; +lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_40 = lean_ctor_get(x_27, 0); +x_41 = lean_ctor_get(x_27, 1); +lean_inc(x_41); +lean_inc(x_40); +lean_dec(x_27); +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_39; +uint8_t x_43; +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); -lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); +lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_39 = !lean_is_exclusive(x_19); -if (x_39 == 0) +lean_dec(x_1); +x_43 = !lean_is_exclusive(x_21); +if (x_43 == 0) { -return x_19; +return x_21; } else { -lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_40 = lean_ctor_get(x_19, 0); -x_41 = lean_ctor_get(x_19, 1); -lean_inc(x_41); -lean_inc(x_40); -lean_dec(x_19); -x_42 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_42, 0, x_40); -lean_ctor_set(x_42, 1, x_41); -return x_42; +lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_44 = lean_ctor_get(x_21, 0); +x_45 = lean_ctor_get(x_21, 1); +lean_inc(x_45); +lean_inc(x_44); +lean_dec(x_21); +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; } } } @@ -18986,9 +16316,9 @@ static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_w _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__1; -x_2 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__2; -x_3 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__3; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__6; +x_2 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__1; +x_3 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__2; x_4 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4___closed__1; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; @@ -19006,9 +16336,9 @@ static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_w _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__1; -x_2 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__2; -x_3 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__3; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__6; +x_2 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__1; +x_3 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__2; x_4 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4___closed__3; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; @@ -19022,115 +16352,110 @@ x_1 = lean_mk_string_unchecked("=>", 2, 2); return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, uint8_t x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19, lean_object* x_20, lean_object* x_21) { _start: { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; -x_18 = lean_ctor_get(x_1, 0); -lean_inc(x_18); -x_19 = lean_box(0); -lean_inc(x_18); -x_20 = l_Lean_RBNode_insert___at_Lean_NameSet_insert___spec__1(x_2, x_18, x_19); -x_21 = l_Lean_Syntax_getArgs(x_8); -x_22 = lean_array_get_size(x_21); -x_23 = lean_unsigned_to_nat(0u); -x_24 = lean_nat_dec_lt(x_23, x_22); -lean_dec(x_22); -if (x_24 == 0) +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; +x_22 = lean_box(0); +lean_inc(x_2); +x_23 = l_Lean_RBNode_insert___at_Lean_NameSet_insert___spec__1(x_1, x_2, x_22); +x_24 = l_Lean_Syntax_getArgs(x_12); +x_25 = lean_array_get_size(x_24); +x_26 = lean_unsigned_to_nat(0u); +x_27 = lean_nat_dec_lt(x_26, x_25); +lean_dec(x_25); +if (x_27 == 0) { -lean_object* x_25; -lean_dec(x_21); -x_25 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__3(x_1, x_3, x_4, x_18, x_5, x_6, x_7, x_20, x_9, x_19, x_11, x_12, x_13, x_14, x_15, x_16, x_17); -lean_dec(x_18); -return x_25; +lean_object* x_28; +lean_dec(x_24); +x_28 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__3(x_3, x_4, x_5, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_23, x_13, x_22, x_15, x_16, x_17, x_18, x_19, x_20, x_21); +return x_28; } else { -lean_object* x_26; uint8_t x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; -x_26 = lean_ctor_get(x_15, 5); -lean_inc(x_26); -x_27 = 0; -x_28 = l_Lean_SourceInfo_fromRef(x_26, x_27); -lean_dec(x_26); -x_29 = lean_st_ref_get(x_16, x_17); -x_30 = !lean_is_exclusive(x_29); -if (x_30 == 0) +lean_object* x_29; uint8_t x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; +x_29 = lean_ctor_get(x_19, 5); +lean_inc(x_29); +x_30 = 0; +x_31 = l_Lean_SourceInfo_fromRef(x_29, x_30); +lean_dec(x_29); +x_32 = lean_st_ref_get(x_20, x_21); +x_33 = !lean_is_exclusive(x_32); +if (x_33 == 0) { -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_31 = lean_ctor_get(x_29, 1); -x_32 = lean_ctor_get(x_29, 0); -lean_dec(x_32); -x_33 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4___closed__1; -lean_inc(x_28); -lean_ctor_set_tag(x_29, 2); -lean_ctor_set(x_29, 1, x_33); -lean_ctor_set(x_29, 0, x_28); -x_34 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__7; -x_35 = l_Array_append___rarg(x_34, x_21); -lean_dec(x_21); -x_36 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__6; -lean_inc(x_28); -x_37 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_37, 0, x_28); -lean_ctor_set(x_37, 1, x_36); -lean_ctor_set(x_37, 2, x_35); -lean_inc(x_28); -x_38 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_38, 0, x_28); -lean_ctor_set(x_38, 1, x_36); -lean_ctor_set(x_38, 2, x_34); -x_39 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4___closed__5; -lean_inc(x_28); -x_40 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_40, 0, x_28); +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_34 = lean_ctor_get(x_32, 1); +x_35 = lean_ctor_get(x_32, 0); +lean_dec(x_35); +x_36 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4___closed__1; +lean_inc(x_31); +lean_ctor_set_tag(x_32, 2); +lean_ctor_set(x_32, 1, x_36); +lean_ctor_set(x_32, 0, x_31); +x_37 = l_Lean_Elab_Command_instInhabitedStructCtorView___closed__1; +x_38 = l_Array_append___rarg(x_37, x_24); +lean_dec(x_24); +x_39 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__10; +lean_inc(x_31); +x_40 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_40, 0, x_31); lean_ctor_set(x_40, 1, x_39); -x_41 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4___closed__4; -lean_inc(x_28); -x_42 = l_Lean_Syntax_node4(x_28, x_41, x_37, x_38, x_40, x_9); -x_43 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4___closed__2; -x_44 = l_Lean_Syntax_node2(x_28, x_43, x_29, x_42); -x_45 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__3(x_1, x_3, x_4, x_18, x_5, x_6, x_7, x_20, x_44, x_19, x_11, x_12, x_13, x_14, x_15, x_16, x_31); -lean_dec(x_18); -return x_45; +lean_ctor_set(x_40, 2, x_38); +lean_inc(x_31); +x_41 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_41, 0, x_31); +lean_ctor_set(x_41, 1, x_39); +lean_ctor_set(x_41, 2, x_37); +x_42 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4___closed__5; +lean_inc(x_31); +x_43 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_43, 0, x_31); +lean_ctor_set(x_43, 1, x_42); +x_44 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4___closed__4; +lean_inc(x_31); +x_45 = l_Lean_Syntax_node4(x_31, x_44, x_40, x_41, x_43, x_13); +x_46 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4___closed__2; +x_47 = l_Lean_Syntax_node2(x_31, x_46, x_32, x_45); +x_48 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__3(x_3, x_4, x_5, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_23, x_47, x_22, x_15, x_16, x_17, x_18, x_19, x_20, x_34); +return x_48; } 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_29, 1); -lean_inc(x_46); -lean_dec(x_29); -x_47 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4___closed__1; -lean_inc(x_28); -x_48 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_48, 0, x_28); -lean_ctor_set(x_48, 1, x_47); -x_49 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__7; -x_50 = l_Array_append___rarg(x_49, x_21); -lean_dec(x_21); -x_51 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__6; -lean_inc(x_28); -x_52 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_52, 0, x_28); -lean_ctor_set(x_52, 1, x_51); -lean_ctor_set(x_52, 2, x_50); -lean_inc(x_28); -x_53 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_53, 0, x_28); -lean_ctor_set(x_53, 1, x_51); -lean_ctor_set(x_53, 2, x_49); -x_54 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4___closed__5; -lean_inc(x_28); -x_55 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_55, 0, x_28); +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_49 = lean_ctor_get(x_32, 1); +lean_inc(x_49); +lean_dec(x_32); +x_50 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4___closed__1; +lean_inc(x_31); +x_51 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_51, 0, x_31); +lean_ctor_set(x_51, 1, x_50); +x_52 = l_Lean_Elab_Command_instInhabitedStructCtorView___closed__1; +x_53 = l_Array_append___rarg(x_52, x_24); +lean_dec(x_24); +x_54 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__10; +lean_inc(x_31); +x_55 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_55, 0, x_31); lean_ctor_set(x_55, 1, x_54); -x_56 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4___closed__4; -lean_inc(x_28); -x_57 = l_Lean_Syntax_node4(x_28, x_56, x_52, x_53, x_55, x_9); -x_58 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4___closed__2; -x_59 = l_Lean_Syntax_node2(x_28, x_58, x_48, x_57); -x_60 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__3(x_1, x_3, x_4, x_18, x_5, x_6, x_7, x_20, x_59, x_19, x_11, x_12, x_13, x_14, x_15, x_16, x_46); -lean_dec(x_18); -return x_60; +lean_ctor_set(x_55, 2, x_53); +lean_inc(x_31); +x_56 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_56, 0, x_31); +lean_ctor_set(x_56, 1, x_54); +lean_ctor_set(x_56, 2, x_52); +x_57 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4___closed__5; +lean_inc(x_31); +x_58 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_58, 0, x_31); +lean_ctor_set(x_58, 1, x_57); +x_59 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4___closed__4; +lean_inc(x_31); +x_60 = l_Lean_Syntax_node4(x_31, x_59, x_55, x_56, x_58, x_13); +x_61 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4___closed__2; +x_62 = l_Lean_Syntax_node2(x_31, x_61, x_51, x_60); +x_63 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__3(x_3, x_4, x_5, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_23, x_62, x_22, x_15, x_16, x_17, x_18, x_19, x_20, x_49); +return x_63; } } } @@ -19255,11 +16580,11 @@ return x_15; } else { -lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; +lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; x_16 = lean_array_fget(x_1, x_3); x_17 = lean_ctor_get(x_16, 0); lean_inc(x_17); -x_18 = lean_ctor_get_uint8(x_16, sizeof(void*)*8); +x_18 = lean_ctor_get_uint8(x_16, sizeof(void*)*9); x_19 = lean_ctor_get(x_16, 2); lean_inc(x_19); x_20 = lean_ctor_get(x_16, 3); @@ -19272,21 +16597,23 @@ x_23 = lean_ctor_get(x_16, 6); lean_inc(x_23); x_24 = lean_ctor_get(x_16, 7); lean_inc(x_24); -x_25 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f(x_5, x_20); -x_26 = !lean_is_exclusive(x_10); -if (x_26 == 0) +x_25 = lean_ctor_get(x_16, 8); +lean_inc(x_25); +x_26 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f(x_5, x_21); +x_27 = !lean_is_exclusive(x_10); +if (x_27 == 0) { -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_10, 5); -x_28 = l_Lean_replaceRef(x_17, x_27); -lean_dec(x_27); -lean_ctor_set(x_10, 5, x_28); -if (lean_obj_tag(x_25) == 0) +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_10, 5); +x_29 = l_Lean_replaceRef(x_17, x_28); +lean_dec(x_28); +lean_ctor_set(x_10, 5, x_29); +if (lean_obj_tag(x_26) == 0) { -lean_object* x_37; +lean_object* x_38; +lean_dec(x_25); lean_dec(x_24); lean_dec(x_23); -lean_dec(x_22); lean_dec(x_17); lean_inc(x_11); lean_inc(x_10); @@ -19294,23 +16621,24 @@ lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -x_37 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabFieldTypeValue(x_16, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_37) == 0) +x_38 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabFieldTypeValue(x_16, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_38) == 0) { -lean_object* x_38; lean_object* x_39; -x_38 = lean_ctor_get(x_37, 0); -lean_inc(x_38); +lean_object* x_39; lean_object* x_40; x_39 = lean_ctor_get(x_38, 0); lean_inc(x_39); -if (lean_obj_tag(x_39) == 0) -{ -lean_object* x_40; -x_40 = lean_ctor_get(x_38, 1); +x_40 = lean_ctor_get(x_39, 0); lean_inc(x_40); -lean_dec(x_38); if (lean_obj_tag(x_40) == 0) { -lean_object* x_41; lean_object* x_42; lean_object* x_43; +lean_object* x_41; +x_41 = lean_ctor_get(x_39, 1); +lean_inc(x_41); +lean_dec(x_39); +if (lean_obj_tag(x_41) == 0) +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; +lean_dec(x_22); lean_dec(x_21); lean_dec(x_20); lean_dec(x_19); @@ -19319,59 +16647,61 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_41 = lean_ctor_get(x_37, 1); -lean_inc(x_41); -lean_dec(x_37); -x_42 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__2; -x_43 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__3___rarg(x_42, x_6, x_7, x_8, x_9, x_10, x_11, x_41); +x_42 = lean_ctor_get(x_38, 1); +lean_inc(x_42); +lean_dec(x_38); +x_43 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__2; +x_44 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__3___rarg(x_43, x_6, x_7, x_8, x_9, x_10, x_11, x_42); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -return x_43; +return x_44; } else { -lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_44 = lean_ctor_get(x_37, 1); -lean_inc(x_44); -lean_dec(x_37); -x_45 = lean_ctor_get(x_40, 0); +lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_45 = lean_ctor_get(x_38, 1); lean_inc(x_45); -lean_dec(x_40); +lean_dec(x_38); +x_46 = lean_ctor_get(x_41, 0); +lean_inc(x_46); +lean_dec(x_41); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -lean_inc(x_45); -x_46 = lean_infer_type(x_45, x_8, x_9, x_10, x_11, x_44); -if (lean_obj_tag(x_46) == 0) +lean_inc(x_46); +x_47 = lean_infer_type(x_46, x_8, x_9, x_10, x_11, x_45); +if (lean_obj_tag(x_47) == 0) { -lean_object* x_47; lean_object* x_48; lean_object* x_49; uint8_t x_50; lean_object* x_51; -x_47 = lean_ctor_get(x_46, 0); -lean_inc(x_47); -x_48 = lean_ctor_get(x_46, 1); +lean_object* x_48; lean_object* x_49; lean_object* x_50; uint8_t x_51; lean_object* x_52; +x_48 = lean_ctor_get(x_47, 0); lean_inc(x_48); -lean_dec(x_46); -x_49 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__1___boxed), 16, 8); -lean_closure_set(x_49, 0, x_45); -lean_closure_set(x_49, 1, x_20); -lean_closure_set(x_49, 2, x_19); -lean_closure_set(x_49, 3, x_5); -lean_closure_set(x_49, 4, x_3); -lean_closure_set(x_49, 5, x_1); -lean_closure_set(x_49, 6, x_2); -lean_closure_set(x_49, 7, x_4); -x_50 = 0; -x_51 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__1___rarg(x_21, x_18, x_47, x_49, x_50, x_6, x_7, x_8, x_9, x_10, x_11, x_48); -return x_51; +x_49 = lean_ctor_get(x_47, 1); +lean_inc(x_49); +lean_dec(x_47); +x_50 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__1___boxed), 17, 9); +lean_closure_set(x_50, 0, x_46); +lean_closure_set(x_50, 1, x_20); +lean_closure_set(x_50, 2, x_21); +lean_closure_set(x_50, 3, x_19); +lean_closure_set(x_50, 4, x_5); +lean_closure_set(x_50, 5, x_3); +lean_closure_set(x_50, 6, x_1); +lean_closure_set(x_50, 7, x_2); +lean_closure_set(x_50, 8, x_4); +x_51 = 0; +x_52 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__1___rarg(x_22, x_18, x_48, x_50, x_51, x_6, x_7, x_8, x_9, x_10, x_11, x_49); +return x_52; } else { -uint8_t x_52; -lean_dec(x_45); +uint8_t x_53; +lean_dec(x_46); lean_dec(x_10); +lean_dec(x_22); lean_dec(x_21); lean_dec(x_20); lean_dec(x_19); @@ -19385,57 +16715,59 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_52 = !lean_is_exclusive(x_46); -if (x_52 == 0) +x_53 = !lean_is_exclusive(x_47); +if (x_53 == 0) { -return x_46; +return x_47; } else { -lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_53 = lean_ctor_get(x_46, 0); -x_54 = lean_ctor_get(x_46, 1); +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); +lean_inc(x_55); lean_inc(x_54); -lean_inc(x_53); -lean_dec(x_46); -x_55 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_55, 0, x_53); -lean_ctor_set(x_55, 1, x_54); -return x_55; +lean_dec(x_47); +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_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; uint8_t x_60; lean_object* x_61; -x_56 = lean_ctor_get(x_37, 1); -lean_inc(x_56); -lean_dec(x_37); +lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; uint8_t x_61; lean_object* x_62; x_57 = lean_ctor_get(x_38, 1); lean_inc(x_57); lean_dec(x_38); -x_58 = lean_ctor_get(x_39, 0); +x_58 = lean_ctor_get(x_39, 1); lean_inc(x_58); lean_dec(x_39); -x_59 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__2___boxed), 16, 8); -lean_closure_set(x_59, 0, x_20); -lean_closure_set(x_59, 1, x_19); -lean_closure_set(x_59, 2, x_57); -lean_closure_set(x_59, 3, x_5); -lean_closure_set(x_59, 4, x_3); -lean_closure_set(x_59, 5, x_1); -lean_closure_set(x_59, 6, x_2); -lean_closure_set(x_59, 7, x_4); -x_60 = 0; -x_61 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__1___rarg(x_21, x_18, x_58, x_59, x_60, x_6, x_7, x_8, x_9, x_10, x_11, x_56); -return x_61; +x_59 = lean_ctor_get(x_40, 0); +lean_inc(x_59); +lean_dec(x_40); +x_60 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__2___boxed), 17, 9); +lean_closure_set(x_60, 0, x_20); +lean_closure_set(x_60, 1, x_21); +lean_closure_set(x_60, 2, x_19); +lean_closure_set(x_60, 3, x_58); +lean_closure_set(x_60, 4, x_5); +lean_closure_set(x_60, 5, x_3); +lean_closure_set(x_60, 6, x_1); +lean_closure_set(x_60, 7, x_2); +lean_closure_set(x_60, 8, x_4); +x_61 = 0; +x_62 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__1___rarg(x_22, x_18, x_59, x_60, x_61, x_6, x_7, x_8, x_9, x_10, x_11, x_57); +return x_62; } } else { -uint8_t x_62; +uint8_t x_63; lean_dec(x_10); +lean_dec(x_22); lean_dec(x_21); lean_dec(x_20); lean_dec(x_19); @@ -19449,149 +16781,158 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_62 = !lean_is_exclusive(x_37); -if (x_62 == 0) +x_63 = !lean_is_exclusive(x_38); +if (x_63 == 0) { -return x_37; +return x_38; } else { -lean_object* x_63; lean_object* x_64; lean_object* x_65; -x_63 = lean_ctor_get(x_37, 0); -x_64 = lean_ctor_get(x_37, 1); +lean_object* x_64; lean_object* x_65; lean_object* x_66; +x_64 = lean_ctor_get(x_38, 0); +x_65 = lean_ctor_get(x_38, 1); +lean_inc(x_65); lean_inc(x_64); -lean_inc(x_63); -lean_dec(x_37); -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_dec(x_38); +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_dec(x_21); +lean_object* x_67; +lean_dec(x_22); lean_dec(x_19); lean_dec(x_16); -if (lean_obj_tag(x_24) == 0) +x_67 = lean_ctor_get(x_26, 0); +lean_inc(x_67); +lean_dec(x_26); +if (lean_obj_tag(x_25) == 0) { -lean_object* x_66; uint8_t x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; +uint8_t x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; +lean_dec(x_24); lean_dec(x_23); -lean_dec(x_22); +lean_dec(x_20); lean_dec(x_17); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_66 = lean_ctor_get(x_25, 0); -lean_inc(x_66); -lean_dec(x_25); -x_67 = lean_ctor_get_uint8(x_66, sizeof(void*)*4); -lean_dec(x_66); -lean_inc(x_20); -x_68 = l_Lean_MessageData_ofName(x_20); -x_69 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__2; -x_70 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_70, 0, x_69); -lean_ctor_set(x_70, 1, x_68); -x_71 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__4; -x_72 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_72, 0, x_70); -lean_ctor_set(x_72, 1, x_71); -switch (x_67) { +x_68 = lean_ctor_get_uint8(x_67, sizeof(void*)*5); +lean_dec(x_67); +lean_inc(x_21); +x_69 = l_Lean_MessageData_ofName(x_21); +x_70 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__2; +x_71 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_71, 0, x_70); +lean_ctor_set(x_71, 1, x_69); +x_72 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__4; +x_73 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_73, 0, x_71); +lean_ctor_set(x_73, 1, x_72); +switch (x_68) { case 0: { -lean_object* x_73; -lean_dec(x_72); -x_73 = lean_box(0); -x_29 = x_73; -goto block_36; +lean_object* x_74; +lean_dec(x_73); +x_74 = lean_box(0); +x_30 = x_74; +goto block_37; } case 1: { -lean_object* x_74; -lean_dec(x_20); -x_74 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__4___rarg(x_72, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_object* x_75; +lean_dec(x_21); +x_75 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__4___rarg(x_73, 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); -return x_74; +return x_75; } case 2: -{ -lean_object* x_75; -lean_dec(x_20); -x_75 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__5___rarg(x_72, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +{ +lean_object* x_76; +lean_dec(x_21); +x_76 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__5___rarg(x_73, 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); -return x_75; +return x_76; } default: { -lean_object* x_76; lean_object* x_77; -lean_dec(x_72); -lean_dec(x_20); -x_76 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__6; -x_77 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__2___rarg(x_76, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_object* x_77; lean_object* x_78; +lean_dec(x_73); +lean_dec(x_21); +x_77 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__6; +x_78 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__2___rarg(x_77, 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); -return x_77; +return x_78; } } } else { -if (lean_obj_tag(x_23) == 0) +if (lean_obj_tag(x_24) == 0) { -lean_object* x_78; uint8_t x_79; lean_object* x_80; lean_object* x_81; uint8_t x_82; -x_78 = lean_ctor_get(x_25, 0); -lean_inc(x_78); -lean_dec(x_25); -x_79 = lean_ctor_get_uint8(x_78, sizeof(void*)*4); -x_80 = lean_ctor_get(x_24, 0); +lean_object* x_79; lean_object* x_80; lean_object* x_81; uint8_t x_82; lean_object* x_83; uint8_t x_84; +x_79 = lean_ctor_get(x_67, 1); +lean_inc(x_79); +x_80 = lean_ctor_get(x_67, 2); lean_inc(x_80); -lean_dec(x_24); -x_81 = lean_ctor_get(x_78, 0); +x_81 = lean_ctor_get(x_67, 3); lean_inc(x_81); -x_82 = l_Lean_NameSet_contains(x_4, x_81); -lean_dec(x_81); -if (x_82 == 0) +x_82 = lean_ctor_get_uint8(x_67, sizeof(void*)*5); +lean_dec(x_67); +x_83 = lean_ctor_get(x_25, 0); +lean_inc(x_83); +lean_dec(x_25); +x_84 = l_Lean_NameSet_contains(x_4, x_79); +if (x_84 == 0) { -lean_object* x_83; -x_83 = lean_box(x_79); -switch (lean_obj_tag(x_83)) { +lean_object* x_85; +x_85 = lean_box(x_82); +switch (lean_obj_tag(x_85)) { case 0: { -lean_object* x_84; +lean_object* x_86; +lean_dec(x_83); +lean_dec(x_81); lean_dec(x_80); -lean_dec(x_78); -lean_dec(x_22); +lean_dec(x_79); +lean_dec(x_23); +lean_dec(x_20); lean_dec(x_17); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_84 = lean_box(0); -x_29 = x_84; -goto block_36; +x_86 = lean_box(0); +x_30 = x_86; +goto block_37; } case 3: { -lean_object* x_85; lean_object* x_86; +lean_object* x_87; lean_object* x_88; +lean_dec(x_83); +lean_dec(x_81); lean_dec(x_80); -lean_dec(x_78); -lean_dec(x_22); +lean_dec(x_79); +lean_dec(x_23); +lean_dec(x_21); lean_dec(x_20); lean_dec(x_17); lean_dec(x_5); @@ -19599,102 +16940,105 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_85 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__6; -x_86 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__2___rarg(x_85, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_87 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__6; +x_88 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__2___rarg(x_87, 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); -return x_86; +return x_88; } default: { -lean_object* x_87; lean_object* x_88; -lean_dec(x_83); -lean_dec(x_20); -x_87 = lean_box(0); -x_88 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4(x_78, x_4, x_17, x_5, x_3, x_1, x_2, x_22, x_80, x_87, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_22); +lean_object* x_89; lean_object* x_90; +lean_dec(x_85); +lean_dec(x_21); +x_89 = lean_box(0); +x_90 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4(x_4, x_79, x_81, x_17, x_20, x_80, x_82, x_5, x_3, x_1, x_2, x_23, x_83, x_89, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_23); lean_dec(x_3); -return x_88; +return x_90; } } } else { -lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; +lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; +lean_dec(x_83); +lean_dec(x_81); lean_dec(x_80); -lean_dec(x_78); -lean_dec(x_22); +lean_dec(x_79); +lean_dec(x_23); +lean_dec(x_20); lean_dec(x_17); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -lean_inc(x_20); -x_89 = l_Lean_MessageData_ofName(x_20); -x_90 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__2; -x_91 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_91, 0, x_90); -lean_ctor_set(x_91, 1, x_89); -x_92 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__8; +lean_inc(x_21); +x_91 = l_Lean_MessageData_ofName(x_21); +x_92 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__2; x_93 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_93, 0, x_91); -lean_ctor_set(x_93, 1, x_92); -x_94 = lean_box(x_79); -switch (lean_obj_tag(x_94)) { +lean_ctor_set(x_93, 0, x_92); +lean_ctor_set(x_93, 1, x_91); +x_94 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__8; +x_95 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_95, 0, x_93); +lean_ctor_set(x_95, 1, x_94); +x_96 = lean_box(x_82); +switch (lean_obj_tag(x_96)) { case 0: { -lean_object* x_95; -lean_dec(x_93); -x_95 = lean_box(0); -x_29 = x_95; -goto block_36; +lean_object* x_97; +lean_dec(x_95); +x_97 = lean_box(0); +x_30 = x_97; +goto block_37; } case 3: { -lean_object* x_96; lean_object* x_97; -lean_dec(x_93); -lean_dec(x_20); -x_96 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__6; -x_97 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__2___rarg(x_96, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_object* x_98; lean_object* x_99; +lean_dec(x_95); +lean_dec(x_21); +x_98 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__6; +x_99 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__2___rarg(x_98, 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); -return x_97; +return x_99; } default: { -lean_object* x_98; uint8_t x_99; -lean_dec(x_94); -lean_dec(x_20); -x_98 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_93, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_object* x_100; uint8_t x_101; +lean_dec(x_96); +lean_dec(x_21); +x_100 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_95, 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); -x_99 = !lean_is_exclusive(x_98); -if (x_99 == 0) +x_101 = !lean_is_exclusive(x_100); +if (x_101 == 0) { -return x_98; +return x_100; } else { -lean_object* x_100; lean_object* x_101; lean_object* x_102; -x_100 = lean_ctor_get(x_98, 0); -x_101 = lean_ctor_get(x_98, 1); -lean_inc(x_101); -lean_inc(x_100); -lean_dec(x_98); -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_102; lean_object* x_103; lean_object* x_104; +x_102 = lean_ctor_get(x_100, 0); +x_103 = lean_ctor_get(x_100, 1); +lean_inc(x_103); +lean_inc(x_102); +lean_dec(x_100); +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; } } } @@ -19702,126 +17046,125 @@ return x_102; } else { -lean_object* x_103; uint8_t x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; -lean_dec(x_24); -lean_dec(x_22); +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_dec(x_25); +lean_dec(x_23); +lean_dec(x_20); lean_dec(x_17); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_103 = lean_ctor_get(x_25, 0); -lean_inc(x_103); -lean_dec(x_25); -x_104 = lean_ctor_get_uint8(x_103, sizeof(void*)*4); -lean_dec(x_103); -x_105 = lean_ctor_get(x_23, 0); -lean_inc(x_105); -lean_dec(x_23); -lean_inc(x_20); -x_106 = l_Lean_MessageData_ofName(x_20); -x_107 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__10; -x_108 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_108, 0, x_107); -lean_ctor_set(x_108, 1, x_106); -x_109 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__12; -x_110 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_110, 0, x_108); -lean_ctor_set(x_110, 1, x_109); -switch (x_104) { +x_105 = lean_ctor_get_uint8(x_67, sizeof(void*)*5); +lean_dec(x_67); +x_106 = lean_ctor_get(x_24, 0); +lean_inc(x_106); +lean_dec(x_24); +lean_inc(x_21); +x_107 = l_Lean_MessageData_ofName(x_21); +x_108 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__10; +x_109 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_109, 0, x_108); +lean_ctor_set(x_109, 1, x_107); +x_110 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__12; +x_111 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_111, 0, x_109); +lean_ctor_set(x_111, 1, x_110); +switch (x_105) { case 0: { -lean_object* x_111; -lean_dec(x_110); -lean_dec(x_105); -x_111 = lean_box(0); -x_29 = x_111; -goto block_36; +lean_object* x_112; +lean_dec(x_111); +lean_dec(x_106); +x_112 = lean_box(0); +x_30 = x_112; +goto block_37; } case 1: { -lean_object* x_112; -lean_dec(x_20); -x_112 = l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__6___rarg(x_105, x_110, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_object* x_113; +lean_dec(x_21); +x_113 = l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__6___rarg(x_106, x_111, 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_105); -return x_112; +lean_dec(x_106); +return x_113; } case 2: { -lean_object* x_113; -lean_dec(x_20); -x_113 = l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__8___rarg(x_105, x_110, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_object* x_114; +lean_dec(x_21); +x_114 = l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__8___rarg(x_106, x_111, 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_105); -return x_113; +lean_dec(x_106); +return x_114; } default: { -lean_object* x_114; lean_object* x_115; -lean_dec(x_110); -lean_dec(x_105); -lean_dec(x_20); -x_114 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__6; -x_115 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__2___rarg(x_114, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_object* x_115; lean_object* x_116; +lean_dec(x_111); +lean_dec(x_106); +lean_dec(x_21); +x_115 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__6; +x_116 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__2___rarg(x_115, 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); -return x_115; +return x_116; } } } } } -block_36: +block_37: { -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_29); -x_30 = l_Lean_MessageData_ofName(x_20); -x_31 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__2; -x_32 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_32, 0, x_31); -lean_ctor_set(x_32, 1, x_30); -x_33 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__6; -x_34 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_34, 0, x_32); -lean_ctor_set(x_34, 1, x_33); -x_35 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__1___rarg(x_34, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +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_30); +x_31 = l_Lean_MessageData_ofName(x_21); +x_32 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__2; +x_33 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_31); +x_34 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__6; +x_35 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +x_36 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__1___rarg(x_35, 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); -return x_35; +return x_36; } } else { -lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; uint8_t x_127; lean_object* x_128; uint8_t x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; -x_116 = lean_ctor_get(x_10, 0); -x_117 = lean_ctor_get(x_10, 1); -x_118 = lean_ctor_get(x_10, 2); -x_119 = lean_ctor_get(x_10, 3); -x_120 = lean_ctor_get(x_10, 4); -x_121 = lean_ctor_get(x_10, 5); -x_122 = lean_ctor_get(x_10, 6); -x_123 = lean_ctor_get(x_10, 7); -x_124 = lean_ctor_get(x_10, 8); -x_125 = lean_ctor_get(x_10, 9); -x_126 = lean_ctor_get(x_10, 10); -x_127 = lean_ctor_get_uint8(x_10, sizeof(void*)*12); -x_128 = lean_ctor_get(x_10, 11); -x_129 = lean_ctor_get_uint8(x_10, sizeof(void*)*12 + 1); -lean_inc(x_128); +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; uint8_t x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; +x_117 = lean_ctor_get(x_10, 0); +x_118 = lean_ctor_get(x_10, 1); +x_119 = lean_ctor_get(x_10, 2); +x_120 = lean_ctor_get(x_10, 3); +x_121 = lean_ctor_get(x_10, 4); +x_122 = lean_ctor_get(x_10, 5); +x_123 = lean_ctor_get(x_10, 6); +x_124 = lean_ctor_get(x_10, 7); +x_125 = lean_ctor_get(x_10, 8); +x_126 = lean_ctor_get(x_10, 9); +x_127 = lean_ctor_get(x_10, 10); +x_128 = lean_ctor_get_uint8(x_10, sizeof(void*)*12); +x_129 = lean_ctor_get(x_10, 11); +x_130 = lean_ctor_get_uint8(x_10, sizeof(void*)*12 + 1); +lean_inc(x_129); +lean_inc(x_127); lean_inc(x_126); lean_inc(x_125); lean_inc(x_124); @@ -19832,55 +17175,55 @@ lean_inc(x_120); lean_inc(x_119); lean_inc(x_118); lean_inc(x_117); -lean_inc(x_116); lean_dec(x_10); -x_130 = l_Lean_replaceRef(x_17, x_121); -lean_dec(x_121); -x_131 = lean_alloc_ctor(0, 12, 2); -lean_ctor_set(x_131, 0, x_116); -lean_ctor_set(x_131, 1, x_117); -lean_ctor_set(x_131, 2, x_118); -lean_ctor_set(x_131, 3, x_119); -lean_ctor_set(x_131, 4, x_120); -lean_ctor_set(x_131, 5, x_130); -lean_ctor_set(x_131, 6, x_122); -lean_ctor_set(x_131, 7, x_123); -lean_ctor_set(x_131, 8, x_124); -lean_ctor_set(x_131, 9, x_125); -lean_ctor_set(x_131, 10, x_126); -lean_ctor_set(x_131, 11, x_128); -lean_ctor_set_uint8(x_131, sizeof(void*)*12, x_127); -lean_ctor_set_uint8(x_131, sizeof(void*)*12 + 1, x_129); -if (lean_obj_tag(x_25) == 0) +x_131 = l_Lean_replaceRef(x_17, x_122); +lean_dec(x_122); +x_132 = lean_alloc_ctor(0, 12, 2); +lean_ctor_set(x_132, 0, x_117); +lean_ctor_set(x_132, 1, x_118); +lean_ctor_set(x_132, 2, x_119); +lean_ctor_set(x_132, 3, x_120); +lean_ctor_set(x_132, 4, x_121); +lean_ctor_set(x_132, 5, x_131); +lean_ctor_set(x_132, 6, x_123); +lean_ctor_set(x_132, 7, x_124); +lean_ctor_set(x_132, 8, x_125); +lean_ctor_set(x_132, 9, x_126); +lean_ctor_set(x_132, 10, x_127); +lean_ctor_set(x_132, 11, x_129); +lean_ctor_set_uint8(x_132, sizeof(void*)*12, x_128); +lean_ctor_set_uint8(x_132, sizeof(void*)*12 + 1, x_130); +if (lean_obj_tag(x_26) == 0) { -lean_object* x_140; +lean_object* x_141; +lean_dec(x_25); lean_dec(x_24); lean_dec(x_23); -lean_dec(x_22); lean_dec(x_17); lean_inc(x_11); -lean_inc(x_131); +lean_inc(x_132); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -x_140 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabFieldTypeValue(x_16, x_6, x_7, x_8, x_9, x_131, x_11, x_12); -if (lean_obj_tag(x_140) == 0) +x_141 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabFieldTypeValue(x_16, x_6, x_7, x_8, x_9, x_132, x_11, x_12); +if (lean_obj_tag(x_141) == 0) { -lean_object* x_141; lean_object* x_142; -x_141 = lean_ctor_get(x_140, 0); -lean_inc(x_141); +lean_object* x_142; lean_object* x_143; x_142 = lean_ctor_get(x_141, 0); lean_inc(x_142); -if (lean_obj_tag(x_142) == 0) -{ -lean_object* x_143; -x_143 = lean_ctor_get(x_141, 1); +x_143 = lean_ctor_get(x_142, 0); lean_inc(x_143); -lean_dec(x_141); if (lean_obj_tag(x_143) == 0) { -lean_object* x_144; lean_object* x_145; lean_object* x_146; +lean_object* x_144; +x_144 = lean_ctor_get(x_142, 1); +lean_inc(x_144); +lean_dec(x_142); +if (lean_obj_tag(x_144) == 0) +{ +lean_object* x_145; lean_object* x_146; lean_object* x_147; +lean_dec(x_22); lean_dec(x_21); lean_dec(x_20); lean_dec(x_19); @@ -19889,59 +17232,61 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_144 = lean_ctor_get(x_140, 1); -lean_inc(x_144); -lean_dec(x_140); -x_145 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__2; -x_146 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__3___rarg(x_145, x_6, x_7, x_8, x_9, x_131, x_11, x_144); +x_145 = lean_ctor_get(x_141, 1); +lean_inc(x_145); +lean_dec(x_141); +x_146 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__2; +x_147 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__3___rarg(x_146, x_6, x_7, x_8, x_9, x_132, x_11, x_145); lean_dec(x_11); -lean_dec(x_131); +lean_dec(x_132); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -return x_146; +return x_147; } else { -lean_object* x_147; lean_object* x_148; lean_object* x_149; -x_147 = lean_ctor_get(x_140, 1); -lean_inc(x_147); -lean_dec(x_140); -x_148 = lean_ctor_get(x_143, 0); +lean_object* x_148; lean_object* x_149; lean_object* x_150; +x_148 = lean_ctor_get(x_141, 1); lean_inc(x_148); -lean_dec(x_143); +lean_dec(x_141); +x_149 = lean_ctor_get(x_144, 0); +lean_inc(x_149); +lean_dec(x_144); lean_inc(x_11); -lean_inc(x_131); +lean_inc(x_132); lean_inc(x_9); lean_inc(x_8); -lean_inc(x_148); -x_149 = lean_infer_type(x_148, x_8, x_9, x_131, x_11, x_147); -if (lean_obj_tag(x_149) == 0) +lean_inc(x_149); +x_150 = lean_infer_type(x_149, x_8, x_9, x_132, x_11, x_148); +if (lean_obj_tag(x_150) == 0) { -lean_object* x_150; lean_object* x_151; lean_object* x_152; uint8_t x_153; lean_object* x_154; -x_150 = lean_ctor_get(x_149, 0); -lean_inc(x_150); -x_151 = lean_ctor_get(x_149, 1); +lean_object* x_151; lean_object* x_152; lean_object* x_153; uint8_t x_154; lean_object* x_155; +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_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__1___boxed), 17, 9); +lean_closure_set(x_153, 0, x_149); +lean_closure_set(x_153, 1, x_20); +lean_closure_set(x_153, 2, x_21); +lean_closure_set(x_153, 3, x_19); +lean_closure_set(x_153, 4, x_5); +lean_closure_set(x_153, 5, x_3); +lean_closure_set(x_153, 6, x_1); +lean_closure_set(x_153, 7, x_2); +lean_closure_set(x_153, 8, x_4); +x_154 = 0; +x_155 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__1___rarg(x_22, x_18, x_151, x_153, x_154, x_6, x_7, x_8, x_9, x_132, x_11, x_152); +return x_155; +} +else +{ +lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_dec(x_149); -x_152 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__1___boxed), 16, 8); -lean_closure_set(x_152, 0, x_148); -lean_closure_set(x_152, 1, x_20); -lean_closure_set(x_152, 2, x_19); -lean_closure_set(x_152, 3, x_5); -lean_closure_set(x_152, 4, x_3); -lean_closure_set(x_152, 5, x_1); -lean_closure_set(x_152, 6, x_2); -lean_closure_set(x_152, 7, x_4); -x_153 = 0; -x_154 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__1___rarg(x_21, x_18, x_150, x_152, x_153, x_6, x_7, x_8, x_9, x_131, x_11, x_151); -return x_154; -} -else -{ -lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; -lean_dec(x_148); -lean_dec(x_131); +lean_dec(x_132); +lean_dec(x_22); lean_dec(x_21); lean_dec(x_20); lean_dec(x_19); @@ -19955,59 +17300,61 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_155 = lean_ctor_get(x_149, 0); -lean_inc(x_155); -x_156 = lean_ctor_get(x_149, 1); +x_156 = lean_ctor_get(x_150, 0); lean_inc(x_156); -if (lean_is_exclusive(x_149)) { - lean_ctor_release(x_149, 0); - lean_ctor_release(x_149, 1); - x_157 = x_149; +x_157 = lean_ctor_get(x_150, 1); +lean_inc(x_157); +if (lean_is_exclusive(x_150)) { + lean_ctor_release(x_150, 0); + lean_ctor_release(x_150, 1); + x_158 = x_150; } else { - lean_dec_ref(x_149); - x_157 = lean_box(0); + lean_dec_ref(x_150); + x_158 = lean_box(0); } -if (lean_is_scalar(x_157)) { - x_158 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_158)) { + x_159 = lean_alloc_ctor(1, 2, 0); } else { - x_158 = x_157; + x_159 = x_158; } -lean_ctor_set(x_158, 0, x_155); -lean_ctor_set(x_158, 1, x_156); -return x_158; +lean_ctor_set(x_159, 0, x_156); +lean_ctor_set(x_159, 1, x_157); +return x_159; } } } else { -lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; uint8_t x_163; lean_object* x_164; -x_159 = lean_ctor_get(x_140, 1); -lean_inc(x_159); -lean_dec(x_140); +lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; uint8_t x_164; lean_object* x_165; x_160 = lean_ctor_get(x_141, 1); lean_inc(x_160); lean_dec(x_141); -x_161 = lean_ctor_get(x_142, 0); +x_161 = lean_ctor_get(x_142, 1); lean_inc(x_161); lean_dec(x_142); -x_162 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__2___boxed), 16, 8); -lean_closure_set(x_162, 0, x_20); -lean_closure_set(x_162, 1, x_19); -lean_closure_set(x_162, 2, x_160); -lean_closure_set(x_162, 3, x_5); -lean_closure_set(x_162, 4, x_3); -lean_closure_set(x_162, 5, x_1); -lean_closure_set(x_162, 6, x_2); -lean_closure_set(x_162, 7, x_4); -x_163 = 0; -x_164 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__1___rarg(x_21, x_18, x_161, x_162, x_163, x_6, x_7, x_8, x_9, x_131, x_11, x_159); -return x_164; +x_162 = lean_ctor_get(x_143, 0); +lean_inc(x_162); +lean_dec(x_143); +x_163 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__2___boxed), 17, 9); +lean_closure_set(x_163, 0, x_20); +lean_closure_set(x_163, 1, x_21); +lean_closure_set(x_163, 2, x_19); +lean_closure_set(x_163, 3, x_161); +lean_closure_set(x_163, 4, x_5); +lean_closure_set(x_163, 5, x_3); +lean_closure_set(x_163, 6, x_1); +lean_closure_set(x_163, 7, x_2); +lean_closure_set(x_163, 8, x_4); +x_164 = 0; +x_165 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__1___rarg(x_22, x_18, x_162, x_163, x_164, x_6, x_7, x_8, x_9, x_132, x_11, x_160); +return x_165; } } else { -lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; -lean_dec(x_131); +lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; +lean_dec(x_132); +lean_dec(x_22); lean_dec(x_21); lean_dec(x_20); lean_dec(x_19); @@ -20021,151 +17368,160 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_165 = lean_ctor_get(x_140, 0); -lean_inc(x_165); -x_166 = lean_ctor_get(x_140, 1); +x_166 = lean_ctor_get(x_141, 0); lean_inc(x_166); -if (lean_is_exclusive(x_140)) { - lean_ctor_release(x_140, 0); - lean_ctor_release(x_140, 1); - x_167 = x_140; +x_167 = lean_ctor_get(x_141, 1); +lean_inc(x_167); +if (lean_is_exclusive(x_141)) { + lean_ctor_release(x_141, 0); + lean_ctor_release(x_141, 1); + x_168 = x_141; } else { - lean_dec_ref(x_140); - x_167 = lean_box(0); + lean_dec_ref(x_141); + x_168 = lean_box(0); } -if (lean_is_scalar(x_167)) { - x_168 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_168)) { + x_169 = lean_alloc_ctor(1, 2, 0); } else { - x_168 = x_167; + x_169 = x_168; } -lean_ctor_set(x_168, 0, x_165); -lean_ctor_set(x_168, 1, x_166); -return x_168; +lean_ctor_set(x_169, 0, x_166); +lean_ctor_set(x_169, 1, x_167); +return x_169; } } else { -lean_dec(x_21); +lean_object* x_170; +lean_dec(x_22); lean_dec(x_19); lean_dec(x_16); -if (lean_obj_tag(x_24) == 0) +x_170 = lean_ctor_get(x_26, 0); +lean_inc(x_170); +lean_dec(x_26); +if (lean_obj_tag(x_25) == 0) { -lean_object* x_169; uint8_t x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; +uint8_t x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; +lean_dec(x_24); lean_dec(x_23); -lean_dec(x_22); +lean_dec(x_20); lean_dec(x_17); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_169 = lean_ctor_get(x_25, 0); -lean_inc(x_169); -lean_dec(x_25); -x_170 = lean_ctor_get_uint8(x_169, sizeof(void*)*4); -lean_dec(x_169); -lean_inc(x_20); -x_171 = l_Lean_MessageData_ofName(x_20); -x_172 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__2; -x_173 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_173, 0, x_172); -lean_ctor_set(x_173, 1, x_171); -x_174 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__4; -x_175 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_175, 0, x_173); -lean_ctor_set(x_175, 1, x_174); -switch (x_170) { +x_171 = lean_ctor_get_uint8(x_170, sizeof(void*)*5); +lean_dec(x_170); +lean_inc(x_21); +x_172 = l_Lean_MessageData_ofName(x_21); +x_173 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__2; +x_174 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_174, 0, x_173); +lean_ctor_set(x_174, 1, x_172); +x_175 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__4; +x_176 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_176, 0, x_174); +lean_ctor_set(x_176, 1, x_175); +switch (x_171) { case 0: { -lean_object* x_176; -lean_dec(x_175); -x_176 = lean_box(0); -x_132 = x_176; -goto block_139; +lean_object* x_177; +lean_dec(x_176); +x_177 = lean_box(0); +x_133 = x_177; +goto block_140; } case 1: { -lean_object* x_177; -lean_dec(x_20); -x_177 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__4___rarg(x_175, x_6, x_7, x_8, x_9, x_131, x_11, x_12); +lean_object* x_178; +lean_dec(x_21); +x_178 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__4___rarg(x_176, x_6, x_7, x_8, x_9, x_132, x_11, x_12); lean_dec(x_11); -lean_dec(x_131); +lean_dec(x_132); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -return x_177; +return x_178; } case 2: { -lean_object* x_178; -lean_dec(x_20); -x_178 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__5___rarg(x_175, x_6, x_7, x_8, x_9, x_131, x_11, x_12); +lean_object* x_179; +lean_dec(x_21); +x_179 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__5___rarg(x_176, x_6, x_7, x_8, x_9, x_132, x_11, x_12); lean_dec(x_11); -lean_dec(x_131); +lean_dec(x_132); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -return x_178; +return x_179; } default: { -lean_object* x_179; lean_object* x_180; -lean_dec(x_175); -lean_dec(x_20); -x_179 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__6; -x_180 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__2___rarg(x_179, x_6, x_7, x_8, x_9, x_131, x_11, x_12); +lean_object* x_180; lean_object* x_181; +lean_dec(x_176); +lean_dec(x_21); +x_180 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__6; +x_181 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__2___rarg(x_180, x_6, x_7, x_8, x_9, x_132, x_11, x_12); lean_dec(x_11); -lean_dec(x_131); +lean_dec(x_132); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -return x_180; +return x_181; } } } else { -if (lean_obj_tag(x_23) == 0) +if (lean_obj_tag(x_24) == 0) { -lean_object* x_181; uint8_t x_182; lean_object* x_183; lean_object* x_184; uint8_t x_185; -x_181 = lean_ctor_get(x_25, 0); -lean_inc(x_181); -lean_dec(x_25); -x_182 = lean_ctor_get_uint8(x_181, sizeof(void*)*4); -x_183 = lean_ctor_get(x_24, 0); +lean_object* x_182; lean_object* x_183; lean_object* x_184; uint8_t x_185; lean_object* x_186; uint8_t x_187; +x_182 = lean_ctor_get(x_170, 1); +lean_inc(x_182); +x_183 = lean_ctor_get(x_170, 2); lean_inc(x_183); -lean_dec(x_24); -x_184 = lean_ctor_get(x_181, 0); +x_184 = lean_ctor_get(x_170, 3); lean_inc(x_184); -x_185 = l_Lean_NameSet_contains(x_4, x_184); -lean_dec(x_184); -if (x_185 == 0) +x_185 = lean_ctor_get_uint8(x_170, sizeof(void*)*5); +lean_dec(x_170); +x_186 = lean_ctor_get(x_25, 0); +lean_inc(x_186); +lean_dec(x_25); +x_187 = l_Lean_NameSet_contains(x_4, x_182); +if (x_187 == 0) { -lean_object* x_186; -x_186 = lean_box(x_182); -switch (lean_obj_tag(x_186)) { +lean_object* x_188; +x_188 = lean_box(x_185); +switch (lean_obj_tag(x_188)) { case 0: { -lean_object* x_187; +lean_object* x_189; +lean_dec(x_186); +lean_dec(x_184); lean_dec(x_183); -lean_dec(x_181); -lean_dec(x_22); +lean_dec(x_182); +lean_dec(x_23); +lean_dec(x_20); lean_dec(x_17); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_187 = lean_box(0); -x_132 = x_187; -goto block_139; +x_189 = lean_box(0); +x_133 = x_189; +goto block_140; } case 3: { -lean_object* x_188; lean_object* x_189; +lean_object* x_190; lean_object* x_191; +lean_dec(x_186); +lean_dec(x_184); lean_dec(x_183); -lean_dec(x_181); -lean_dec(x_22); +lean_dec(x_182); +lean_dec(x_23); +lean_dec(x_21); lean_dec(x_20); lean_dec(x_17); lean_dec(x_5); @@ -20173,211 +17529,212 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_188 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__6; -x_189 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__2___rarg(x_188, x_6, x_7, x_8, x_9, x_131, x_11, x_12); +x_190 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__6; +x_191 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__2___rarg(x_190, x_6, x_7, x_8, x_9, x_132, x_11, x_12); lean_dec(x_11); -lean_dec(x_131); +lean_dec(x_132); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -return x_189; +return x_191; } default: { -lean_object* x_190; lean_object* x_191; -lean_dec(x_186); -lean_dec(x_20); -x_190 = lean_box(0); -x_191 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4(x_181, x_4, x_17, x_5, x_3, x_1, x_2, x_22, x_183, x_190, x_6, x_7, x_8, x_9, x_131, x_11, x_12); -lean_dec(x_22); +lean_object* x_192; lean_object* x_193; +lean_dec(x_188); +lean_dec(x_21); +x_192 = lean_box(0); +x_193 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4(x_4, x_182, x_184, x_17, x_20, x_183, x_185, x_5, x_3, x_1, x_2, x_23, x_186, x_192, x_6, x_7, x_8, x_9, x_132, x_11, x_12); +lean_dec(x_23); lean_dec(x_3); -return x_191; +return x_193; } } } else { -lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; +lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; +lean_dec(x_186); +lean_dec(x_184); lean_dec(x_183); -lean_dec(x_181); -lean_dec(x_22); +lean_dec(x_182); +lean_dec(x_23); +lean_dec(x_20); lean_dec(x_17); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -lean_inc(x_20); -x_192 = l_Lean_MessageData_ofName(x_20); -x_193 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__2; -x_194 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_194, 0, x_193); -lean_ctor_set(x_194, 1, x_192); -x_195 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__8; +lean_inc(x_21); +x_194 = l_Lean_MessageData_ofName(x_21); +x_195 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__2; x_196 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_196, 0, x_194); -lean_ctor_set(x_196, 1, x_195); -x_197 = lean_box(x_182); -switch (lean_obj_tag(x_197)) { +lean_ctor_set(x_196, 0, x_195); +lean_ctor_set(x_196, 1, x_194); +x_197 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__8; +x_198 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_198, 0, x_196); +lean_ctor_set(x_198, 1, x_197); +x_199 = lean_box(x_185); +switch (lean_obj_tag(x_199)) { case 0: { -lean_object* x_198; -lean_dec(x_196); -x_198 = lean_box(0); -x_132 = x_198; -goto block_139; +lean_object* x_200; +lean_dec(x_198); +x_200 = lean_box(0); +x_133 = x_200; +goto block_140; } case 3: { -lean_object* x_199; lean_object* x_200; -lean_dec(x_196); -lean_dec(x_20); -x_199 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__6; -x_200 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__2___rarg(x_199, x_6, x_7, x_8, x_9, x_131, x_11, x_12); +lean_object* x_201; lean_object* x_202; +lean_dec(x_198); +lean_dec(x_21); +x_201 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__6; +x_202 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__2___rarg(x_201, x_6, x_7, x_8, x_9, x_132, x_11, x_12); lean_dec(x_11); -lean_dec(x_131); +lean_dec(x_132); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -return x_200; +return x_202; } default: { -lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; -lean_dec(x_197); -lean_dec(x_20); -x_201 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_196, x_6, x_7, x_8, x_9, x_131, x_11, x_12); +lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; +lean_dec(x_199); +lean_dec(x_21); +x_203 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_198, x_6, x_7, x_8, x_9, x_132, x_11, x_12); lean_dec(x_11); -lean_dec(x_131); +lean_dec(x_132); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -x_202 = lean_ctor_get(x_201, 0); -lean_inc(x_202); -x_203 = lean_ctor_get(x_201, 1); -lean_inc(x_203); -if (lean_is_exclusive(x_201)) { - lean_ctor_release(x_201, 0); - lean_ctor_release(x_201, 1); - x_204 = x_201; +x_204 = lean_ctor_get(x_203, 0); +lean_inc(x_204); +x_205 = lean_ctor_get(x_203, 1); +lean_inc(x_205); +if (lean_is_exclusive(x_203)) { + lean_ctor_release(x_203, 0); + lean_ctor_release(x_203, 1); + x_206 = x_203; } else { - lean_dec_ref(x_201); - x_204 = lean_box(0); + lean_dec_ref(x_203); + x_206 = lean_box(0); } -if (lean_is_scalar(x_204)) { - x_205 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_206)) { + x_207 = lean_alloc_ctor(1, 2, 0); } else { - x_205 = x_204; + x_207 = x_206; } -lean_ctor_set(x_205, 0, x_202); -lean_ctor_set(x_205, 1, x_203); -return x_205; +lean_ctor_set(x_207, 0, x_204); +lean_ctor_set(x_207, 1, x_205); +return x_207; } } } } else { -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; lean_object* x_213; -lean_dec(x_24); -lean_dec(x_22); +uint8_t x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; +lean_dec(x_25); +lean_dec(x_23); +lean_dec(x_20); lean_dec(x_17); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_206 = lean_ctor_get(x_25, 0); -lean_inc(x_206); -lean_dec(x_25); -x_207 = lean_ctor_get_uint8(x_206, sizeof(void*)*4); -lean_dec(x_206); -x_208 = lean_ctor_get(x_23, 0); -lean_inc(x_208); -lean_dec(x_23); -lean_inc(x_20); -x_209 = l_Lean_MessageData_ofName(x_20); -x_210 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__10; -x_211 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_211, 0, x_210); -lean_ctor_set(x_211, 1, x_209); -x_212 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__12; -x_213 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_213, 0, x_211); -lean_ctor_set(x_213, 1, x_212); -switch (x_207) { +x_208 = lean_ctor_get_uint8(x_170, sizeof(void*)*5); +lean_dec(x_170); +x_209 = lean_ctor_get(x_24, 0); +lean_inc(x_209); +lean_dec(x_24); +lean_inc(x_21); +x_210 = l_Lean_MessageData_ofName(x_21); +x_211 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__10; +x_212 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_212, 0, x_211); +lean_ctor_set(x_212, 1, x_210); +x_213 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__12; +x_214 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_214, 0, x_212); +lean_ctor_set(x_214, 1, x_213); +switch (x_208) { case 0: { -lean_object* x_214; -lean_dec(x_213); -lean_dec(x_208); -x_214 = lean_box(0); -x_132 = x_214; -goto block_139; +lean_object* x_215; +lean_dec(x_214); +lean_dec(x_209); +x_215 = lean_box(0); +x_133 = x_215; +goto block_140; } case 1: { -lean_object* x_215; -lean_dec(x_20); -x_215 = l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__6___rarg(x_208, x_213, x_6, x_7, x_8, x_9, x_131, x_11, x_12); +lean_object* x_216; +lean_dec(x_21); +x_216 = l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__6___rarg(x_209, x_214, x_6, x_7, x_8, x_9, x_132, x_11, x_12); lean_dec(x_11); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_208); -return x_215; +lean_dec(x_209); +return x_216; } case 2: { -lean_object* x_216; -lean_dec(x_20); -x_216 = l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__8___rarg(x_208, x_213, x_6, x_7, x_8, x_9, x_131, x_11, x_12); +lean_object* x_217; +lean_dec(x_21); +x_217 = l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__8___rarg(x_209, x_214, x_6, x_7, x_8, x_9, x_132, x_11, x_12); lean_dec(x_11); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_208); -return x_216; +lean_dec(x_209); +return x_217; } default: { -lean_object* x_217; lean_object* x_218; -lean_dec(x_213); -lean_dec(x_208); -lean_dec(x_20); -x_217 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__6; -x_218 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__2___rarg(x_217, x_6, x_7, x_8, x_9, x_131, x_11, x_12); +lean_object* x_218; lean_object* x_219; +lean_dec(x_214); +lean_dec(x_209); +lean_dec(x_21); +x_218 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__6; +x_219 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__2___rarg(x_218, x_6, x_7, x_8, x_9, x_132, x_11, x_12); lean_dec(x_11); -lean_dec(x_131); +lean_dec(x_132); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -return x_218; +return x_219; } } } } } -block_139: +block_140: { -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_132); -x_133 = l_Lean_MessageData_ofName(x_20); -x_134 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__2; -x_135 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_135, 0, x_134); -lean_ctor_set(x_135, 1, x_133); -x_136 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__6; -x_137 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_137, 0, x_135); -lean_ctor_set(x_137, 1, x_136); -x_138 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__1___rarg(x_137, x_6, x_7, x_8, x_9, x_131, x_11, x_12); +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_dec(x_133); +x_134 = l_Lean_MessageData_ofName(x_21); +x_135 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__2; +x_136 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_136, 0, x_135); +lean_ctor_set(x_136, 1, x_134); +x_137 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__6; +x_138 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_138, 0, x_136); +lean_ctor_set(x_138, 1, x_137); +x_139 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__1___rarg(x_138, x_6, x_7, x_8, x_9, x_132, x_11, x_12); lean_dec(x_11); -lean_dec(x_131); +lean_dec(x_132); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -return x_138; +return x_139; } } } @@ -20508,22 +17865,56 @@ lean_dec(x_1); return x_10; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___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: { -lean_object* x_17; -x_17 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_5); -return x_17; +lean_object* x_18; +x_18 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +lean_dec(x_6); +return x_18; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_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, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___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: { -lean_object* x_17; -x_17 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_5); -return x_17; +lean_object* x_18; +x_18 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +lean_dec(x_6); +return x_18; } } LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__3___boxed(lean_object** _args) { @@ -20544,14 +17935,18 @@ lean_object* x_14 = _args[13]; lean_object* x_15 = _args[14]; lean_object* x_16 = _args[15]; lean_object* x_17 = _args[16]; +lean_object* x_18 = _args[17]; +lean_object* x_19 = _args[18]; +lean_object* x_20 = _args[19]; _start: { -lean_object* x_18; -x_18 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); -lean_dec(x_10); -lean_dec(x_5); -lean_dec(x_4); -return x_18; +uint8_t x_21; lean_object* x_22; +x_21 = lean_unbox(x_6); +lean_dec(x_6); +x_22 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__3(x_1, x_2, x_3, x_4, x_5, x_21, 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_13); +lean_dec(x_8); +return x_22; } } LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4___boxed(lean_object** _args) { @@ -20572,14 +17967,20 @@ 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]; _start: { -lean_object* x_18; -x_18 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); -lean_dec(x_10); -lean_dec(x_8); -lean_dec(x_5); -return x_18; +uint8_t x_22; lean_object* x_23; +x_22 = lean_unbox(x_7); +lean_dec(x_7); +x_23 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_22, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20, x_21); +lean_dec(x_14); +lean_dec(x_12); +lean_dec(x_9); +return x_23; } } LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_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, lean_object* x_8, lean_object* x_9, lean_object* x_10) { @@ -20730,7 +18131,7 @@ if (x_11 == 0) lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_dec(x_4); x_12 = lean_array_uget(x_1, x_2); -x_13 = lean_ctor_get(x_12, 2); +x_13 = lean_ctor_get(x_12, 3); lean_inc(x_13); lean_inc(x_9); lean_inc(x_8); @@ -20746,7 +18147,7 @@ x_16 = lean_ctor_get(x_14, 1); lean_inc(x_16); lean_dec(x_14); x_17 = l_Lean_Expr_collectFVars(x_15, x_5, x_6, x_7, x_8, x_9, x_16); -x_18 = lean_ctor_get(x_12, 3); +x_18 = lean_ctor_get(x_12, 4); lean_inc(x_18); lean_dec(x_12); if (lean_obj_tag(x_18) == 0) @@ -21105,7 +18506,7 @@ static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_r lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = lean_box(0); x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_removeUnused___closed__3; -x_3 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; +x_3 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__1; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_2); lean_ctor_set(x_4, 1, x_1); @@ -21571,7 +18972,7 @@ return x_13; } else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; lean_object* x_21; lean_object* x_22; +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; lean_object* x_22; lean_object* x_23; x_14 = lean_array_uget(x_4, x_3); x_15 = lean_unsigned_to_nat(0u); x_16 = lean_array_uset(x_4, x_3, x_15); @@ -21581,148 +18982,155 @@ x_18 = lean_ctor_get(x_14, 1); lean_inc(x_18); x_19 = lean_ctor_get(x_14, 2); lean_inc(x_19); -x_20 = lean_ctor_get_uint8(x_14, sizeof(void*)*4); -x_21 = lean_ctor_get(x_14, 3); -lean_inc(x_21); +x_20 = lean_ctor_get(x_14, 3); +lean_inc(x_20); +x_21 = lean_ctor_get_uint8(x_14, sizeof(void*)*5); +x_22 = lean_ctor_get(x_14, 4); +lean_inc(x_22); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_19); +lean_inc(x_20); lean_inc(x_1); -x_22 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParamFVar(x_1, x_19, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_22) == 0) +x_23 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParamFVar(x_1, x_20, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_23) == 0) { -if (lean_obj_tag(x_21) == 0) +if (lean_obj_tag(x_22) == 0) { -lean_object* x_23; size_t x_24; size_t x_25; lean_object* x_26; +lean_object* x_24; size_t x_25; size_t x_26; lean_object* x_27; +lean_dec(x_20); lean_dec(x_19); lean_dec(x_18); lean_dec(x_17); -x_23 = lean_ctor_get(x_22, 1); -lean_inc(x_23); -lean_dec(x_22); -x_24 = 1; -x_25 = lean_usize_add(x_3, x_24); -x_26 = lean_array_uset(x_16, x_3, x_14); -x_3 = x_25; -x_4 = x_26; -x_11 = x_23; +x_24 = lean_ctor_get(x_23, 1); +lean_inc(x_24); +lean_dec(x_23); +x_25 = 1; +x_26 = lean_usize_add(x_3, x_25); +x_27 = lean_array_uset(x_16, x_3, x_14); +x_3 = x_26; +x_4 = x_27; +x_11 = x_24; goto _start; } else { -uint8_t x_28; -x_28 = !lean_is_exclusive(x_14); -if (x_28 == 0) +uint8_t x_29; +x_29 = !lean_is_exclusive(x_14); +if (x_29 == 0) { -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; -x_29 = lean_ctor_get(x_14, 3); -lean_dec(x_29); -x_30 = lean_ctor_get(x_14, 2); +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; +x_30 = lean_ctor_get(x_14, 4); lean_dec(x_30); -x_31 = lean_ctor_get(x_14, 1); +x_31 = lean_ctor_get(x_14, 3); lean_dec(x_31); -x_32 = lean_ctor_get(x_14, 0); +x_32 = lean_ctor_get(x_14, 2); lean_dec(x_32); -x_33 = lean_ctor_get(x_22, 1); -lean_inc(x_33); -lean_dec(x_22); -x_34 = !lean_is_exclusive(x_21); -if (x_34 == 0) -{ -lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; size_t x_39; size_t x_40; lean_object* x_41; -x_35 = lean_ctor_get(x_21, 0); -lean_inc(x_1); -x_36 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27(x_1, x_35, x_5, x_6, x_7, x_8, x_9, x_10, 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); -lean_ctor_set(x_21, 0, x_37); -x_39 = 1; -x_40 = lean_usize_add(x_3, x_39); -x_41 = lean_array_uset(x_16, x_3, x_14); -x_3 = x_40; -x_4 = x_41; -x_11 = x_38; +x_33 = lean_ctor_get(x_14, 1); +lean_dec(x_33); +x_34 = lean_ctor_get(x_14, 0); +lean_dec(x_34); +x_35 = lean_ctor_get(x_23, 1); +lean_inc(x_35); +lean_dec(x_23); +x_36 = !lean_is_exclusive(x_22); +if (x_36 == 0) +{ +lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; size_t x_41; size_t x_42; lean_object* x_43; +x_37 = lean_ctor_get(x_22, 0); +lean_inc(x_1); +x_38 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27(x_1, x_37, x_5, x_6, x_7, x_8, x_9, x_10, x_35); +x_39 = lean_ctor_get(x_38, 0); +lean_inc(x_39); +x_40 = lean_ctor_get(x_38, 1); +lean_inc(x_40); +lean_dec(x_38); +lean_ctor_set(x_22, 0, x_39); +x_41 = 1; +x_42 = lean_usize_add(x_3, x_41); +x_43 = lean_array_uset(x_16, x_3, x_14); +x_3 = x_42; +x_4 = x_43; +x_11 = x_40; goto _start; } else { -lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; size_t x_48; size_t x_49; lean_object* x_50; -x_43 = lean_ctor_get(x_21, 0); -lean_inc(x_43); -lean_dec(x_21); -lean_inc(x_1); -x_44 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27(x_1, x_43, x_5, x_6, x_7, x_8, x_9, x_10, x_33); -x_45 = lean_ctor_get(x_44, 0); +lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; size_t x_50; size_t x_51; lean_object* x_52; +x_45 = lean_ctor_get(x_22, 0); lean_inc(x_45); -x_46 = lean_ctor_get(x_44, 1); -lean_inc(x_46); -lean_dec(x_44); -x_47 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_47, 0, x_45); -lean_ctor_set(x_14, 3, x_47); -x_48 = 1; -x_49 = lean_usize_add(x_3, x_48); -x_50 = lean_array_uset(x_16, x_3, x_14); -x_3 = x_49; -x_4 = x_50; -x_11 = x_46; +lean_dec(x_22); +lean_inc(x_1); +x_46 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27(x_1, x_45, x_5, x_6, x_7, x_8, x_9, x_10, x_35); +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_alloc_ctor(1, 1, 0); +lean_ctor_set(x_49, 0, x_47); +lean_ctor_set(x_14, 4, x_49); +x_50 = 1; +x_51 = lean_usize_add(x_3, x_50); +x_52 = lean_array_uset(x_16, x_3, x_14); +x_3 = x_51; +x_4 = x_52; +x_11 = x_48; goto _start; } } else { -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; size_t x_60; size_t x_61; lean_object* x_62; +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; size_t x_62; size_t x_63; lean_object* x_64; lean_dec(x_14); -x_52 = lean_ctor_get(x_22, 1); -lean_inc(x_52); -lean_dec(x_22); -x_53 = lean_ctor_get(x_21, 0); -lean_inc(x_53); -if (lean_is_exclusive(x_21)) { - lean_ctor_release(x_21, 0); - x_54 = x_21; +x_54 = lean_ctor_get(x_23, 1); +lean_inc(x_54); +lean_dec(x_23); +x_55 = lean_ctor_get(x_22, 0); +lean_inc(x_55); +if (lean_is_exclusive(x_22)) { + lean_ctor_release(x_22, 0); + x_56 = x_22; } else { - lean_dec_ref(x_21); - x_54 = lean_box(0); + lean_dec_ref(x_22); + x_56 = lean_box(0); } lean_inc(x_1); -x_55 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27(x_1, x_53, x_5, x_6, x_7, x_8, x_9, x_10, x_52); -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); -if (lean_is_scalar(x_54)) { - x_58 = lean_alloc_ctor(1, 1, 0); +x_57 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27(x_1, x_55, x_5, x_6, x_7, x_8, x_9, x_10, x_54); +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); +if (lean_is_scalar(x_56)) { + x_60 = lean_alloc_ctor(1, 1, 0); } else { - x_58 = x_54; + x_60 = x_56; } -lean_ctor_set(x_58, 0, x_56); -x_59 = lean_alloc_ctor(0, 4, 1); -lean_ctor_set(x_59, 0, x_17); -lean_ctor_set(x_59, 1, x_18); -lean_ctor_set(x_59, 2, x_19); -lean_ctor_set(x_59, 3, x_58); -lean_ctor_set_uint8(x_59, sizeof(void*)*4, x_20); -x_60 = 1; -x_61 = lean_usize_add(x_3, x_60); -x_62 = lean_array_uset(x_16, x_3, x_59); -x_3 = x_61; -x_4 = x_62; -x_11 = x_57; +lean_ctor_set(x_60, 0, x_58); +x_61 = lean_alloc_ctor(0, 5, 1); +lean_ctor_set(x_61, 0, x_17); +lean_ctor_set(x_61, 1, x_18); +lean_ctor_set(x_61, 2, x_19); +lean_ctor_set(x_61, 3, x_20); +lean_ctor_set(x_61, 4, x_60); +lean_ctor_set_uint8(x_61, sizeof(void*)*5, x_21); +x_62 = 1; +x_63 = lean_usize_add(x_3, x_62); +x_64 = lean_array_uset(x_16, x_3, x_61); +x_3 = x_63; +x_4 = x_64; +x_11 = x_59; goto _start; } } } else { -uint8_t x_64; -lean_dec(x_21); +uint8_t x_66; +lean_dec(x_22); +lean_dec(x_20); lean_dec(x_19); lean_dec(x_18); lean_dec(x_17); @@ -21733,23 +19141,23 @@ lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_1); -x_64 = !lean_is_exclusive(x_22); -if (x_64 == 0) +x_66 = !lean_is_exclusive(x_23); +if (x_66 == 0) { -return x_22; +return x_23; } else { -lean_object* x_65; lean_object* x_66; lean_object* x_67; -x_65 = lean_ctor_get(x_22, 0); -x_66 = lean_ctor_get(x_22, 1); -lean_inc(x_66); -lean_inc(x_65); -lean_dec(x_22); -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_67; lean_object* x_68; lean_object* x_69; +x_67 = lean_ctor_get(x_23, 0); +x_68 = lean_ctor_get(x_23, 1); +lean_inc(x_68); +lean_inc(x_67); +lean_dec(x_23); +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; } } } @@ -22059,7 +19467,7 @@ else lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_27; lean_object* x_28; lean_dec(x_6); x_17 = lean_array_uget(x_3, x_5); -x_27 = lean_ctor_get(x_17, 2); +x_27 = lean_ctor_get(x_17, 3); lean_inc(x_27); lean_inc(x_13); lean_inc(x_12); @@ -22135,7 +19543,7 @@ lean_inc(x_51); x_52 = lean_ctor_get(x_50, 1); lean_inc(x_52); lean_dec(x_50); -x_53 = lean_ctor_get(x_17, 1); +x_53 = lean_ctor_get(x_17, 2); lean_inc(x_53); lean_dec(x_17); x_54 = l_Lean_MessageData_ofName(x_53); @@ -22148,7 +19556,7 @@ lean_ctor_set_tag(x_42, 7); lean_ctor_set(x_42, 1, x_56); lean_ctor_set(x_42, 0, x_46); x_57 = l_Lean_MessageData_ofExpr(x_29); -x_58 = l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__4; +x_58 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3; lean_ctor_set_tag(x_38, 7); lean_ctor_set(x_38, 1, x_57); lean_ctor_set(x_38, 0, x_58); @@ -22359,7 +19767,7 @@ lean_inc(x_98); x_99 = lean_ctor_get(x_97, 1); lean_inc(x_99); lean_dec(x_97); -x_100 = lean_ctor_get(x_17, 1); +x_100 = lean_ctor_get(x_17, 2); lean_inc(x_100); lean_dec(x_17); x_101 = l_Lean_MessageData_ofName(x_100); @@ -22372,7 +19780,7 @@ lean_ctor_set_tag(x_42, 7); lean_ctor_set(x_42, 1, x_104); lean_ctor_set(x_42, 0, x_103); x_105 = l_Lean_MessageData_ofExpr(x_29); -x_106 = l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__4; +x_106 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3; lean_ctor_set_tag(x_38, 7); lean_ctor_set(x_38, 1, x_105); lean_ctor_set(x_38, 0, x_106); @@ -22623,7 +20031,7 @@ lean_inc(x_152); x_153 = lean_ctor_get(x_151, 1); lean_inc(x_153); lean_dec(x_151); -x_154 = lean_ctor_get(x_17, 1); +x_154 = lean_ctor_get(x_17, 2); lean_inc(x_154); lean_dec(x_17); x_155 = l_Lean_MessageData_ofName(x_154); @@ -22641,7 +20049,7 @@ x_159 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_159, 0, x_157); lean_ctor_set(x_159, 1, x_158); x_160 = l_Lean_MessageData_ofExpr(x_29); -x_161 = l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__4; +x_161 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3; lean_ctor_set_tag(x_38, 7); lean_ctor_set(x_38, 1, x_160); lean_ctor_set(x_38, 0, x_161); @@ -22905,7 +20313,7 @@ lean_inc(x_211); x_212 = lean_ctor_get(x_210, 1); lean_inc(x_212); lean_dec(x_210); -x_213 = lean_ctor_get(x_17, 1); +x_213 = lean_ctor_get(x_17, 2); lean_inc(x_213); lean_dec(x_17); x_214 = l_Lean_MessageData_ofName(x_213); @@ -22928,7 +20336,7 @@ if (lean_is_scalar(x_206)) { lean_ctor_set(x_218, 0, x_216); lean_ctor_set(x_218, 1, x_217); x_219 = l_Lean_MessageData_ofExpr(x_29); -x_220 = l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__4; +x_220 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3; x_221 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_221, 0, x_220); lean_ctor_set(x_221, 1, x_219); @@ -23205,7 +20613,7 @@ lean_inc(x_275); x_276 = lean_ctor_get(x_274, 1); lean_inc(x_276); lean_dec(x_274); -x_277 = lean_ctor_get(x_17, 1); +x_277 = lean_ctor_get(x_17, 2); lean_inc(x_277); lean_dec(x_17); x_278 = l_Lean_MessageData_ofName(x_277); @@ -23228,7 +20636,7 @@ if (lean_is_scalar(x_270)) { lean_ctor_set(x_282, 0, x_280); lean_ctor_set(x_282, 1, x_281); x_283 = l_Lean_MessageData_ofExpr(x_29); -x_284 = l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__4; +x_284 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3; if (lean_is_scalar(x_266)) { x_285 = lean_alloc_ctor(7, 2, 0); } else { @@ -23665,7 +21073,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_co _start: { lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_11 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; +x_11 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__1; x_12 = lean_st_mk_ref(x_11, x_10); x_13 = lean_ctor_get(x_12, 0); lean_inc(x_13); @@ -23735,40 +21143,316 @@ lean_dec(x_3); return x_11; } } -LEAN_EXPORT uint8_t l___private_Lean_Elab_Structure_0__Lean_Elab_Command_isPropCandidate(lean_object* x_1) { -_start: +LEAN_EXPORT uint8_t l___private_Lean_Elab_Structure_0__Lean_Elab_Command_isPropCandidate(lean_object* x_1) { +_start: +{ +uint8_t x_2; +x_2 = l_Array_isEmpty___rarg(x_1); +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; +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_isPropCandidate___boxed(lean_object* x_1) { +_start: +{ +uint8_t x_2; lean_object* x_3; +x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_isPropCandidate(x_1); +lean_dec(x_1); +x_3 = lean_box(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +uint8_t x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_14 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_isPropCandidate(x_1); +x_15 = l_Lean_Elab_Command_mkResultUniverse(x_2, x_3, x_14); +x_16 = l_Lean_Level_mvarId_x21(x_4); +x_17 = l_Lean_assignLevelMVar___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___spec__1(x_16, x_15, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +x_18 = lean_ctor_get(x_17, 1); +lean_inc(x_18); +lean_dec(x_17); +x_19 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_5, x_7, x_8, x_9, x_10, x_11, x_12, x_18); +return x_19; +} +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__7; +x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__4; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("updateResultingUniverse us: ", 28, 28); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__2; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(", r: ", 5, 5); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__4; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(", rOffset: ", 11, 11); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__6; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___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: +{ +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_2); +lean_inc(x_1); +x_13 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields(x_1, x_2, x_3, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_13) == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_13, 1); +lean_inc(x_15); +lean_dec(x_13); +x_16 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__1; +x_17 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_16, x_6, x_7, x_8, x_9, x_10, x_11, x_15); +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_unbox(x_18); +lean_dec(x_18); +if (x_19 == 0) +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_17, 1); +lean_inc(x_20); +lean_dec(x_17); +x_21 = lean_box(0); +x_22 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__1(x_3, x_14, x_2, x_1, x_4, x_21, 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); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_1); +lean_dec(x_2); +return x_22; +} +else +{ +uint8_t x_23; +x_23 = !lean_is_exclusive(x_17); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; 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; +x_24 = lean_ctor_get(x_17, 1); +x_25 = lean_ctor_get(x_17, 0); +lean_dec(x_25); +lean_inc(x_14); +x_26 = lean_array_to_list(x_14); +x_27 = lean_box(0); +x_28 = l_List_mapTR_loop___at_Lean_Meta_Match_mkMatcher___spec__6(x_26, x_27); +x_29 = l_Lean_MessageData_ofList(x_28); +x_30 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__3; +lean_ctor_set_tag(x_17, 7); +lean_ctor_set(x_17, 1, x_29); +lean_ctor_set(x_17, 0, x_30); +x_31 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__5; +x_32 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_32, 0, x_17); +lean_ctor_set(x_32, 1, x_31); +lean_inc(x_1); +x_33 = l_Lean_MessageData_ofLevel(x_1); +x_34 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_34, 0, x_32); +lean_ctor_set(x_34, 1, x_33); +x_35 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__7; +x_36 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_36, 0, x_34); +lean_ctor_set(x_36, 1, x_35); +lean_inc(x_2); +x_37 = l___private_Init_Data_Repr_0__Nat_reprFast(x_2); +x_38 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_38, 0, x_37); +x_39 = l_Lean_MessageData_ofFormat(x_38); +x_40 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_40, 0, x_36); +lean_ctor_set(x_40, 1, x_39); +x_41 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3; +x_42 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_42, 0, x_40); +lean_ctor_set(x_42, 1, x_41); +x_43 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_16, x_42, x_6, x_7, x_8, x_9, x_10, x_11, x_24); +x_44 = lean_ctor_get(x_43, 0); +lean_inc(x_44); +x_45 = lean_ctor_get(x_43, 1); +lean_inc(x_45); +lean_dec(x_43); +x_46 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__1(x_3, x_14, x_2, x_1, x_4, x_44, x_6, x_7, x_8, x_9, x_10, x_11, x_45); +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_44); +lean_dec(x_1); +lean_dec(x_2); +return x_46; +} +else +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; +x_47 = lean_ctor_get(x_17, 1); +lean_inc(x_47); +lean_dec(x_17); +lean_inc(x_14); +x_48 = lean_array_to_list(x_14); +x_49 = lean_box(0); +x_50 = l_List_mapTR_loop___at_Lean_Meta_Match_mkMatcher___spec__6(x_48, x_49); +x_51 = l_Lean_MessageData_ofList(x_50); +x_52 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__3; +x_53 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_53, 0, x_52); +lean_ctor_set(x_53, 1, x_51); +x_54 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__5; +x_55 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_55, 0, x_53); +lean_ctor_set(x_55, 1, x_54); +lean_inc(x_1); +x_56 = l_Lean_MessageData_ofLevel(x_1); +x_57 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_57, 0, x_55); +lean_ctor_set(x_57, 1, x_56); +x_58 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__7; +x_59 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_59, 0, x_57); +lean_ctor_set(x_59, 1, x_58); +lean_inc(x_2); +x_60 = l___private_Init_Data_Repr_0__Nat_reprFast(x_2); +x_61 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_61, 0, x_60); +x_62 = l_Lean_MessageData_ofFormat(x_61); +x_63 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_63, 0, x_59); +lean_ctor_set(x_63, 1, x_62); +x_64 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3; +x_65 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_65, 0, x_63); +lean_ctor_set(x_65, 1, x_64); +x_66 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_16, x_65, x_6, x_7, x_8, x_9, x_10, x_11, x_47); +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___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__1(x_3, x_14, x_2, x_1, x_4, x_67, x_6, x_7, x_8, x_9, x_10, x_11, x_68); +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_67); +lean_dec(x_1); +lean_dec(x_2); +return x_69; +} +} +} +else { -uint8_t x_2; -x_2 = l_Array_isEmpty___rarg(x_1); -if (x_2 == 0) +uint8_t x_70; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_70 = !lean_is_exclusive(x_13); +if (x_70 == 0) { -uint8_t x_3; -x_3 = 1; -return x_3; +return x_13; } else { -uint8_t x_4; -x_4 = 0; -return x_4; -} +lean_object* x_71; lean_object* x_72; lean_object* x_73; +x_71 = lean_ctor_get(x_13, 0); +x_72 = lean_ctor_get(x_13, 1); +lean_inc(x_72); +lean_inc(x_71); +lean_dec(x_13); +x_73 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_73, 0, x_71); +lean_ctor_set(x_73, 1, x_72); +return x_73; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_isPropCandidate___boxed(lean_object* x_1) { -_start: -{ -uint8_t x_2; lean_object* x_3; -x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_isPropCandidate(x_1); -lean_dec(x_1); -x_3 = lean_box(x_2); -return x_3; } } static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("failed to compute resulting universe level of structure, provide universe explicitly", 84, 84); +x_1 = lean_mk_string_unchecked("failed to compute resulting universe level of inductive datatype, provide universe explicitly: ", 95, 95); return x_1; } } @@ -23794,7 +21478,7 @@ lean_inc(x_2); x_10 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getResultUniverse(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); if (lean_obj_tag(x_10) == 0) { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; x_11 = lean_ctor_get(x_10, 0); lean_inc(x_11); x_12 = lean_ctor_get(x_10, 1); @@ -23804,94 +21488,57 @@ x_13 = lean_unsigned_to_nat(0u); x_14 = l_Lean_Level_getOffsetAux(x_11, x_13); x_15 = l_Lean_Level_getLevelOffset(x_11); lean_dec(x_11); -if (lean_obj_tag(x_15) == 5) -{ -lean_object* x_16; lean_object* x_17; -x_16 = lean_ctor_get(x_15, 0); -lean_inc(x_16); -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_14); -x_17 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields(x_15, x_14, x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_12); -if (lean_obj_tag(x_17) == 0) -{ -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; -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_17, 1); -lean_inc(x_19); -lean_dec(x_17); -x_20 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_isPropCandidate(x_1); -x_21 = l_Lean_Elab_Command_mkResultUniverse(x_18, x_14, x_20); -lean_dec(x_14); -x_22 = l_Lean_assignLevelMVar___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_updateResultingUniverse___spec__1(x_16, x_21, x_3, x_4, x_5, x_6, x_7, x_8, x_19); -x_23 = lean_ctor_get(x_22, 1); -lean_inc(x_23); -lean_dec(x_22); -x_24 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_23); -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_24; -} -else +x_16 = l_Lean_Level_isMVar(x_15); +if (x_16 == 0) { -uint8_t x_25; -lean_dec(x_16); +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_dec(x_14); +lean_dec(x_2); +x_17 = l_Lean_MessageData_ofLevel(x_15); +x_18 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___closed__2; +x_19 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set(x_19, 1, x_17); +x_20 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3; +x_21 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_21, 0, x_19); +lean_ctor_set(x_21, 1, x_20); +x_22 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_21, x_3, x_4, x_5, x_6, x_7, x_8, x_12); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_25 = !lean_is_exclusive(x_17); -if (x_25 == 0) +x_23 = !lean_is_exclusive(x_22); +if (x_23 == 0) { -return x_17; +return x_22; } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_17, 0); -x_27 = lean_ctor_get(x_17, 1); -lean_inc(x_27); -lean_inc(x_26); -lean_dec(x_17); -x_28 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_28, 0, x_26); -lean_ctor_set(x_28, 1, x_27); -return x_28; -} +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_22, 0); +x_25 = lean_ctor_get(x_22, 1); +lean_inc(x_25); +lean_inc(x_24); +lean_dec(x_22); +x_26 = lean_alloc_ctor(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_29; lean_object* x_30; -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_2); -x_29 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___closed__2; -x_30 = l_Lean_throwError___at_Lean_Elab_Term_tryPostponeIfHasMVars___spec__1(x_29, x_3, x_4, x_5, x_6, x_7, x_8, x_12); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -return x_30; +lean_object* x_27; lean_object* x_28; +x_27 = lean_box(0); +x_28 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2(x_15, x_14, x_1, x_2, x_27, x_3, x_4, x_5, x_6, x_7, x_8, x_12); +return x_28; } } else { -uint8_t x_31; +uint8_t x_29; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -23899,26 +21546,54 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_31 = !lean_is_exclusive(x_10); -if (x_31 == 0) +x_29 = !lean_is_exclusive(x_10); +if (x_29 == 0) { return x_10; } else { -lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_32 = lean_ctor_get(x_10, 0); -x_33 = lean_ctor_get(x_10, 1); -lean_inc(x_33); -lean_inc(x_32); +lean_object* x_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_dec(x_10); -x_34 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_34, 0, x_32); -lean_ctor_set(x_34, 1, x_33); -return x_34; +x_32 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_31); +return x_32; +} +} +} } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; +x_14 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +return x_14; } } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; +x_13 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_5); +lean_dec(x_3); +return x_13; +} } LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, 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: @@ -24168,7 +21843,7 @@ if (x_12 == 0) { lean_object* x_13; lean_object* x_14; lean_object* x_15; x_13 = lean_array_uget(x_1, x_2); -x_14 = lean_ctor_get(x_13, 2); +x_14 = lean_ctor_get(x_13, 3); lean_inc(x_14); lean_dec(x_13); lean_inc(x_10); @@ -24237,7 +21912,7 @@ static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_c { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_removeUnused___closed__3; -x_2 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; +x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__1; x_3 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_1); @@ -24602,7 +22277,7 @@ goto block_57; block_57: { lean_object* x_16; lean_object* x_17; -x_16 = lean_ctor_get(x_15, 2); +x_16 = lean_ctor_get(x_15, 3); lean_inc(x_16); lean_inc(x_9); lean_inc(x_8); @@ -24634,7 +22309,7 @@ x_25 = lean_array_mk(x_20); x_26 = lean_expr_abstract(x_22, x_25); lean_dec(x_25); lean_dec(x_22); -x_27 = lean_ctor_get_uint8(x_15, sizeof(void*)*4); +x_27 = lean_ctor_get_uint8(x_15, sizeof(void*)*5); lean_dec(x_15); x_28 = lean_box(x_27); if (lean_obj_tag(x_28) == 2) @@ -24681,7 +22356,7 @@ x_41 = lean_array_mk(x_40); x_42 = lean_expr_abstract(x_37, x_41); lean_dec(x_41); lean_dec(x_37); -x_43 = lean_ctor_get_uint8(x_15, sizeof(void*)*4); +x_43 = lean_ctor_get_uint8(x_15, sizeof(void*)*5); lean_dec(x_15); x_44 = lean_box(x_43); if (lean_obj_tag(x_44) == 2) @@ -25144,7 +22819,59 @@ x_6 = lean_mk_projections(x_1, x_2, x_3, x_5); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___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; lean_object* x_7; +x_5 = lean_ctor_get(x_1, 0); +x_6 = lean_ctor_get(x_1, 1); +x_7 = lean_ctor_get(x_5, 2); +lean_inc(x_7); +lean_dec(x_5); +lean_ctor_set(x_1, 1, x_2); +lean_ctor_set(x_1, 0, x_7); +{ +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_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_9 = lean_ctor_get(x_1, 0); +x_10 = lean_ctor_get(x_1, 1); +lean_inc(x_10); +lean_inc(x_9); +lean_dec(x_1); +x_11 = lean_ctor_get(x_9, 2); +lean_inc(x_11); +lean_dec(x_9); +x_12 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_12, 0, x_11); +lean_ctor_set(x_12, 1, x_2); +x_1 = x_10; +x_2 = x_12; +goto _start; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; @@ -25226,19 +22953,19 @@ return x_29; } } } -LEAN_EXPORT lean_object* l_Lean_throwKernelException___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___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_EXPORT lean_object* l_Lean_throwKernelException___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___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; lean_object* x_10; lean_object* x_11; x_9 = lean_ctor_get(x_6, 2); lean_inc(x_9); x_10 = l_Lean_KernelException_toMessageData(x_1, x_9); -x_11 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__3(x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_11 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__4(x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_6); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_ofExceptKernelException___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___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_ofExceptKernelException___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { if (lean_obj_tag(x_1) == 0) @@ -25247,7 +22974,7 @@ lean_object* x_9; lean_object* x_10; x_9 = lean_ctor_get(x_1, 0); lean_inc(x_9); lean_dec(x_1); -x_10 = l_Lean_throwKernelException___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__2(x_9, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_10 = l_Lean_throwKernelException___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__3(x_9, x_2, x_3, x_4, x_5, x_6, x_7, x_8); return x_10; } else @@ -25265,7 +22992,60 @@ return x_12; } } } -LEAN_EXPORT lean_object* l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___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) { +static lean_object* _init_l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__2; +x_2 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_2, 0, x_1); +lean_ctor_set(x_2, 1, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__2; +x_2 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_2, 0, x_1); +lean_ctor_set(x_2, 1, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__2; +x_2 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_2, 0, x_1); +lean_ctor_set(x_2, 1, x_1); +lean_ctor_set(x_2, 2, x_1); +lean_ctor_set(x_2, 3, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__2; +x_2 = l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__2; +x_3 = l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__3; +x_4 = lean_alloc_ctor(0, 7, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_2); +lean_ctor_set(x_4, 3, x_2); +lean_ctor_set(x_4, 4, x_2); +lean_ctor_set(x_4, 5, x_3); +lean_ctor_set(x_4, 6, x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; @@ -25283,7 +23063,7 @@ x_13 = lean_ctor_get(x_10, 4); lean_dec(x_13); x_14 = lean_ctor_get(x_10, 0); lean_dec(x_14); -x_15 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__4; +x_15 = l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__1; lean_ctor_set(x_10, 4, x_15); lean_ctor_set(x_10, 0, x_1); x_16 = lean_st_ref_set(x_7, x_10, x_11); @@ -25302,7 +23082,7 @@ if (x_21 == 0) lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; x_22 = lean_ctor_get(x_19, 1); lean_dec(x_22); -x_23 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__7; +x_23 = l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__4; lean_ctor_set(x_19, 1, x_23); x_24 = lean_st_ref_set(x_5, x_19, x_20); x_25 = !lean_is_exclusive(x_24); @@ -25340,7 +23120,7 @@ lean_inc(x_33); lean_inc(x_32); lean_inc(x_31); lean_dec(x_19); -x_35 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__7; +x_35 = l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__4; x_36 = lean_alloc_ctor(0, 5, 0); lean_ctor_set(x_36, 0, x_31); lean_ctor_set(x_36, 1, x_35); @@ -25383,7 +23163,7 @@ lean_inc(x_44); lean_inc(x_43); lean_inc(x_42); lean_dec(x_10); -x_47 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__4; +x_47 = l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__1; x_48 = lean_alloc_ctor(0, 7, 0); lean_ctor_set(x_48, 0, x_1); lean_ctor_set(x_48, 1, x_42); @@ -25421,101 +23201,571 @@ if (lean_is_exclusive(x_52)) { lean_dec_ref(x_52); x_58 = lean_box(0); } -x_59 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__7; -if (lean_is_scalar(x_58)) { - x_60 = lean_alloc_ctor(0, 5, 0); -} else { - x_60 = x_58; +x_59 = l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__4; +if (lean_is_scalar(x_58)) { + x_60 = lean_alloc_ctor(0, 5, 0); +} else { + x_60 = x_58; +} +lean_ctor_set(x_60, 0, x_54); +lean_ctor_set(x_60, 1, x_59); +lean_ctor_set(x_60, 2, x_55); +lean_ctor_set(x_60, 3, x_56); +lean_ctor_set(x_60, 4, x_57); +x_61 = lean_st_ref_set(x_5, x_60, x_53); +x_62 = lean_ctor_get(x_61, 1); +lean_inc(x_62); +if (lean_is_exclusive(x_61)) { + lean_ctor_release(x_61, 0); + lean_ctor_release(x_61, 1); + x_63 = x_61; +} else { + lean_dec_ref(x_61); + x_63 = lean_box(0); +} +x_64 = lean_box(0); +if (lean_is_scalar(x_63)) { + x_65 = lean_alloc_ctor(0, 2, 0); +} else { + x_65 = x_63; +} +lean_ctor_set(x_65, 0, x_64); +lean_ctor_set(x_65, 1, x_62); +return x_65; +} +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___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; uint8_t x_7; size_t x_8; size_t x_9; +x_6 = lean_array_uget(x_1, x_2); +x_7 = l_Lean_Elab_Command_StructFieldInfo_isFromParent(x_6); +x_8 = 1; +x_9 = lean_usize_add(x_2, x_8); +if (x_7 == 0) +{ +lean_object* x_10; +x_10 = lean_array_push(x_4, x_6); +x_2 = x_9; +x_4 = x_10; +goto _start; +} +else +{ +lean_dec(x_6); +x_2 = x_9; +goto _start; +} +} +else +{ +return x_4; +} +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__7(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; lean_object* x_17; +lean_dec(x_5); +x_15 = lean_array_uget(x_2, x_4); +x_16 = lean_ctor_get(x_15, 3); +lean_inc(x_16); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +x_17 = l_Lean_Meta_isProof(x_16, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_17) == 0) +{ +lean_object* x_18; uint8_t x_19; +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_unbox(x_18); +lean_dec(x_18); +if (x_19 == 0) +{ +uint8_t x_20; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_1); +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; +x_21 = lean_ctor_get(x_17, 0); +lean_dec(x_21); +x_22 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_22, 0, x_15); +x_23 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_23, 0, x_22); +x_24 = lean_box(0); +x_25 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +lean_ctor_set(x_17, 0, x_25); +return x_17; +} +else +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_26 = lean_ctor_get(x_17, 1); +lean_inc(x_26); +lean_dec(x_17); +x_27 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_27, 0, x_15); +x_28 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_28, 0, x_27); +x_29 = lean_box(0); +x_30 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_30); +lean_ctor_set(x_31, 1, x_26); +return x_31; +} +} +else +{ +lean_object* x_32; size_t x_33; size_t x_34; +lean_dec(x_15); +x_32 = lean_ctor_get(x_17, 1); +lean_inc(x_32); +lean_dec(x_17); +x_33 = 1; +x_34 = lean_usize_add(x_4, x_33); +lean_inc(x_1); +{ +size_t _tmp_3 = x_34; +lean_object* _tmp_4 = x_1; +lean_object* _tmp_11 = x_32; +x_4 = _tmp_3; +x_5 = _tmp_4; +x_12 = _tmp_11; +} +goto _start; +} +} +else +{ +uint8_t x_36; +lean_dec(x_15); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_1); +x_36 = !lean_is_exclusive(x_17); +if (x_36 == 0) +{ +return x_17; +} +else +{ +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_17, 0); +x_38 = lean_ctor_get(x_17, 1); +lean_inc(x_38); +lean_inc(x_37); +lean_dec(x_17); +x_39 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_39, 0, x_37); +lean_ctor_set(x_39, 1, x_38); +return x_39; +} +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___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; uint8_t x_14; lean_object* x_15; lean_object* x_16; +x_11 = lean_array_get_size(x_1); +x_12 = lean_box(0); +x_13 = lean_unsigned_to_nat(0u); +x_14 = lean_nat_dec_lt(x_13, x_11); +x_15 = lean_st_ref_get(x_9, x_10); +if (x_14 == 0) +{ +lean_object* x_35; +lean_dec(x_11); +x_35 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__1; +x_16 = x_35; +goto block_34; +} +else +{ +uint8_t x_36; +x_36 = lean_nat_dec_le(x_11, x_11); +if (x_36 == 0) +{ +lean_object* x_37; +lean_dec(x_11); +x_37 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__1; +x_16 = x_37; +goto block_34; +} +else +{ +size_t x_38; size_t x_39; lean_object* x_40; lean_object* x_41; +x_38 = 0; +x_39 = lean_usize_of_nat(x_11); +lean_dec(x_11); +x_40 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__1; +x_41 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__6(x_1, x_38, x_39, x_40); +x_16 = x_41; +goto block_34; +} +} +block_34: +{ +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_17 = lean_ctor_get(x_15, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_15, 1); +lean_inc(x_18); +lean_dec(x_15); +x_19 = lean_array_to_list(x_16); +x_20 = l_List_mapTR_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__1(x_19, x_12); +x_21 = lean_ctor_get(x_17, 0); +lean_inc(x_21); +lean_dec(x_17); +x_22 = lean_ctor_get(x_2, 0); +lean_inc(x_22); +lean_dec(x_2); +x_23 = lean_ctor_get(x_22, 4); +lean_inc(x_23); +x_24 = lean_ctor_get_uint8(x_22, sizeof(void*)*12); +lean_dec(x_22); +x_25 = lean_mk_projections(x_21, x_23, x_20, x_24); +lean_inc(x_8); +lean_inc(x_4); +x_26 = l_Lean_ofExceptKernelException___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__2(x_25, x_4, x_5, x_6, x_7, x_8, x_9, x_18); +if (lean_obj_tag(x_26) == 0) +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_26, 0); +lean_inc(x_27); +x_28 = lean_ctor_get(x_26, 1); +lean_inc(x_28); +lean_dec(x_26); +x_29 = l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5(x_27, x_4, x_5, x_6, x_7, x_8, x_9, x_28); +lean_dec(x_8); +lean_dec(x_4); +return x_29; +} +else +{ +uint8_t x_30; +lean_dec(x_8); +lean_dec(x_4); +x_30 = !lean_is_exclusive(x_26); +if (x_30 == 0) +{ +return x_26; +} +else +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_31 = lean_ctor_get(x_26, 0); +x_32 = lean_ctor_get(x_26, 1); +lean_inc(x_32); +lean_inc(x_31); +lean_dec(x_26); +x_33 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_33, 0, x_31); +lean_ctor_set(x_33, 1, x_32); +return x_33; +} +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___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; +x_10 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_10, 0, x_1); +lean_ctor_set(x_10, 1, x_9); +return x_10; +} } -lean_ctor_set(x_60, 0, x_54); -lean_ctor_set(x_60, 1, x_59); -lean_ctor_set(x_60, 2, x_55); -lean_ctor_set(x_60, 3, x_56); -lean_ctor_set(x_60, 4, x_57); -x_61 = lean_st_ref_set(x_5, x_60, x_53); -x_62 = lean_ctor_get(x_61, 1); -lean_inc(x_62); -if (lean_is_exclusive(x_61)) { - lean_ctor_release(x_61, 0); - lean_ctor_release(x_61, 1); - x_63 = x_61; -} else { - lean_dec_ref(x_61); - x_63 = lean_box(0); +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("failed to generate projections for 'Prop' structure, field '", 60, 60); +return x_1; } -x_64 = lean_box(0); -if (lean_is_scalar(x_63)) { - x_65 = lean_alloc_ctor(0, 2, 0); -} else { - x_65 = x_63; } -lean_ctor_set(x_65, 0, x_64); -lean_ctor_set(x_65, 1, x_62); -return x_65; +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("' is not a proof", 16, 16); +return x_1; +} } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___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; -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); -x_15 = lean_mk_projections(x_14, x_1, x_2, x_3); +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; uint8_t x_11; +x_10 = lean_ctor_get(x_1, 5); +lean_inc(x_10); +x_11 = l_Lean_Expr_isProp(x_10); +lean_dec(x_10); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; +x_12 = lean_box(0); +x_13 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___lambda__1(x_2, x_1, x_12, 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); +return x_13; +} +else +{ +lean_object* x_14; size_t x_15; size_t x_16; lean_object* x_17; lean_object* x_18; lean_object* x_56; lean_object* x_57; +x_14 = lean_box(0); +x_15 = lean_array_size(x_2); +x_16 = 0; +x_56 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___closed__1; lean_inc(x_8); -lean_inc(x_4); -x_16 = l_Lean_ofExceptKernelException___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__1(x_15, x_4, x_5, x_6, x_7, x_8, x_9, x_13); -if (lean_obj_tag(x_16) == 0) +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_57 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__7(x_56, x_2, x_15, x_16, 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_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_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__4(x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_18); +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_58, 0); +lean_inc(x_59); +lean_dec(x_58); +if (lean_obj_tag(x_59) == 0) +{ +lean_object* x_60; +x_60 = lean_ctor_get(x_57, 1); +lean_inc(x_60); +lean_dec(x_57); +x_17 = x_14; +x_18 = x_60; +goto block_55; +} +else +{ +lean_object* x_61; lean_object* x_62; +x_61 = lean_ctor_get(x_57, 1); +lean_inc(x_61); +lean_dec(x_57); +x_62 = lean_ctor_get(x_59, 0); +lean_inc(x_62); +lean_dec(x_59); +x_17 = x_62; +x_18 = x_61; +goto block_55; +} +} +else +{ +uint8_t x_63; lean_dec(x_8); -lean_dec(x_4); -return x_19; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_1); +x_63 = !lean_is_exclusive(x_57); +if (x_63 == 0) +{ +return x_57; } else { -uint8_t x_20; +lean_object* x_64; lean_object* x_65; lean_object* x_66; +x_64 = lean_ctor_get(x_57, 0); +x_65 = lean_ctor_get(x_57, 1); +lean_inc(x_65); +lean_inc(x_64); +lean_dec(x_57); +x_66 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_66, 0, x_64); +lean_ctor_set(x_66, 1, x_65); +return x_66; +} +} +block_55: +{ +if (lean_obj_tag(x_17) == 0) +{ +lean_object* x_19; lean_object* x_20; +x_19 = lean_box(0); +x_20 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___lambda__1(x_2, x_1, x_19, x_3, x_4, x_5, x_6, x_7, x_8, x_18); lean_dec(x_8); -lean_dec(x_4); -x_20 = !lean_is_exclusive(x_16); -if (x_20 == 0) +lean_dec(x_6); +lean_dec(x_5); +return x_20; +} +else { -return x_16; +uint8_t x_21; +lean_dec(x_1); +x_21 = !lean_is_exclusive(x_17); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; +x_22 = lean_ctor_get(x_17, 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_22); +x_25 = 1; +x_26 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___closed__1; +x_27 = l_Lean_Name_toString(x_24, x_25, x_26); +lean_ctor_set_tag(x_17, 3); +lean_ctor_set(x_17, 0, x_27); +x_28 = l_Lean_MessageData_ofFormat(x_17); +x_29 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___closed__2; +x_30 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_30, 0, x_29); +lean_ctor_set(x_30, 1, x_28); +x_31 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___closed__4; +x_32 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_31); +x_33 = l_Lean_throwErrorAt___at___private_Lean_Elab_Binders_0__Lean_Elab_Term_elabBinderViews_loop___spec__1(x_23, x_32, x_3, x_4, x_5, x_6, x_7, x_8, x_18); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_23); +x_34 = !lean_is_exclusive(x_33); +if (x_34 == 0) +{ +return x_33; } else { -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_16, 0); -x_22 = lean_ctor_get(x_16, 1); -lean_inc(x_22); -lean_inc(x_21); -lean_dec(x_16); -x_23 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_23, 0, x_21); -lean_ctor_set(x_23, 1, x_22); -return x_23; +lean_object* x_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_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; +} +} +else +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_38 = lean_ctor_get(x_17, 0); +lean_inc(x_38); +lean_dec(x_17); +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 = 1; +x_42 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___closed__1; +x_43 = l_Lean_Name_toString(x_40, x_41, x_42); +x_44 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_44, 0, x_43); +x_45 = l_Lean_MessageData_ofFormat(x_44); +x_46 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___closed__2; +x_47 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_47, 0, x_46); +lean_ctor_set(x_47, 1, x_45); +x_48 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___closed__4; +x_49 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_49, 0, x_47); +lean_ctor_set(x_49, 1, x_48); +x_50 = l_Lean_throwErrorAt___at___private_Lean_Elab_Binders_0__Lean_Elab_Term_elabBinderViews_loop___spec__1(x_39, x_49, x_3, x_4, x_5, x_6, x_7, x_8, x_18); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_39); +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(1, 2, 0); +} else { + x_54 = x_53; +} +lean_ctor_set(x_54, 0, x_51); +lean_ctor_set(x_54, 1, x_52); +return x_54; +} +} } } } } -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; -x_9 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -25524,11 +23774,11 @@ lean_dec(x_3); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_throwKernelException___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___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_EXPORT lean_object* l_Lean_throwKernelException___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___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_throwKernelException___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_throwKernelException___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_7); lean_dec(x_5); lean_dec(x_4); @@ -25536,11 +23786,11 @@ lean_dec(x_3); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_ofExceptKernelException___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___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_ofExceptKernelException___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___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) { _start: { lean_object* x_9; -x_9 = l_Lean_ofExceptKernelException___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_ofExceptKernelException___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_7); lean_dec(x_5); lean_dec(x_4); @@ -25548,11 +23798,11 @@ lean_dec(x_3); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___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_EXPORT lean_object* l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; -x_9 = l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -25562,18 +23812,71 @@ lean_dec(x_2); return x_9; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_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_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___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___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__6(x_1, x_5, x_6, x_4); +lean_dec(x_1); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___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) { _start: { -uint8_t x_11; lean_object* x_12; -x_11 = lean_unbox(x_3); +size_t x_13; size_t x_14; lean_object* x_15; +x_13 = lean_unbox_usize(x_3); lean_dec(x_3); -x_12 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections(x_1, x_2, x_11, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_14 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_15 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__7(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_2); +return x_15; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, 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_Structure_0__Lean_Elab_Command_addProjections___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); lean_dec(x_6); lean_dec(x_5); -return x_12; +lean_dec(x_3); +lean_dec(x_1); +return x_11; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_10; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections(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_2); +return x_10; } } static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___closed__1() { @@ -25598,7 +23901,7 @@ static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Str lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__1; x_2 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___closed__1; -x_3 = lean_unsigned_to_nat(730u); +x_3 = lean_unsigned_to_nat(801u); x_4 = lean_unsigned_to_nat(21u); x_5 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -25619,7 +23922,7 @@ static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Str lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__1; x_2 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___closed__1; -x_3 = lean_unsigned_to_nat(729u); +x_3 = lean_unsigned_to_nat(800u); x_4 = lean_unsigned_to_nat(23u); x_5 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___closed__4; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -25633,1985 +23936,2462 @@ uint8_t x_12; x_12 = lean_usize_dec_eq(x_2, x_3); if (x_12 == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_25; lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; lean_object* x_48; uint8_t x_49; uint8_t x_50; +lean_object* x_13; lean_object* x_14; lean_object* x_25; uint8_t x_44; uint8_t x_45; uint8_t x_46; x_13 = lean_array_uget(x_1, x_2); -x_44 = lean_ctor_get(x_13, 0); -lean_inc(x_44); -x_45 = lean_ctor_get(x_13, 1); -lean_inc(x_45); -x_46 = lean_ctor_get(x_13, 2); -lean_inc(x_46); -x_47 = lean_ctor_get_uint8(x_13, sizeof(void*)*4); -if (lean_is_exclusive(x_13)) { - lean_ctor_release(x_13, 0); - lean_ctor_release(x_13, 1); - lean_ctor_release(x_13, 2); - lean_ctor_release(x_13, 3); - x_48 = x_13; -} else { - lean_dec_ref(x_13); - x_48 = lean_box(0); -} -x_49 = 2; -x_50 = l_Lean_Elab_Command_instDecidableEqStructFieldKind(x_47, x_49); -if (x_50 == 0) +x_44 = lean_ctor_get_uint8(x_13, sizeof(void*)*5); +x_45 = 2; +x_46 = l_Lean_Elab_Command_instDecidableEqStructFieldKind(x_44, x_45); +if (x_46 == 0) { -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_51 = lean_st_ref_get(x_10, x_11); -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); +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_47 = lean_st_ref_get(x_10, x_11); +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_ctor_get(x_48, 0); +lean_inc(x_50); +lean_dec(x_48); +x_51 = lean_ctor_get(x_13, 3); +lean_inc(x_51); lean_inc(x_7); -x_55 = l_Lean_Meta_getFVarLocalDecl(x_46, x_7, x_8, x_9, x_10, x_53); -if (lean_obj_tag(x_55) == 0) +x_52 = l_Lean_Meta_getFVarLocalDecl(x_51, x_7, x_8, x_9, x_10, x_49); +if (lean_obj_tag(x_52) == 0) { -uint8_t x_56; -x_56 = !lean_is_exclusive(x_55); -if (x_56 == 0) +uint8_t x_53; +x_53 = !lean_is_exclusive(x_52); +if (x_53 == 0) { -lean_object* x_57; lean_object* x_58; lean_object* x_59; -x_57 = lean_ctor_get(x_55, 0); -x_58 = lean_ctor_get(x_55, 1); +lean_object* x_54; lean_object* x_55; lean_object* x_56; +x_54 = lean_ctor_get(x_52, 0); +x_55 = lean_ctor_get(x_52, 1); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -x_59 = lean_infer_type(x_46, x_7, x_8, x_9, x_10, x_58); -if (lean_obj_tag(x_59) == 0) +x_56 = lean_infer_type(x_51, x_7, x_8, x_9, x_10, x_55); +if (lean_obj_tag(x_56) == 0) { -lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; uint8_t x_64; uint8_t x_65; lean_object* x_66; lean_object* x_67; -x_60 = lean_ctor_get(x_59, 0); +lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; uint8_t x_63; uint8_t x_64; lean_object* x_65; lean_object* x_66; +x_57 = lean_ctor_get(x_56, 0); +lean_inc(x_57); +x_58 = lean_ctor_get(x_56, 1); +lean_inc(x_58); +if (lean_is_exclusive(x_56)) { + lean_ctor_release(x_56, 0); + lean_ctor_release(x_56, 1); + x_59 = x_56; +} else { + lean_dec_ref(x_56); + x_59 = lean_box(0); +} +x_60 = lean_ctor_get(x_13, 1); lean_inc(x_60); -x_61 = lean_ctor_get(x_59, 1); +x_61 = lean_ctor_get(x_13, 2); lean_inc(x_61); -if (lean_is_exclusive(x_59)) { - lean_ctor_release(x_59, 0); - lean_ctor_release(x_59, 1); - x_62 = x_59; +lean_dec(x_13); +x_62 = 3; +x_63 = l_Lean_Elab_Command_instDecidableEqStructFieldKind(x_44, x_62); +x_64 = l_Lean_LocalDecl_binderInfo(x_54); +lean_dec(x_54); +x_65 = l_Lean_Expr_getAutoParamTactic_x3f(x_57); +lean_dec(x_57); +if (x_63 == 0) +{ +lean_object* x_71; lean_object* x_72; lean_object* x_73; +lean_dec(x_59); +lean_dec(x_50); +x_71 = lean_box(0); +x_72 = lean_alloc_ctor(0, 4, 1); +lean_ctor_set(x_72, 0, x_60); +lean_ctor_set(x_72, 1, x_61); +lean_ctor_set(x_72, 2, x_71); +lean_ctor_set(x_72, 3, x_65); +lean_ctor_set_uint8(x_72, sizeof(void*)*4, x_64); +x_73 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_73, 0, x_72); +lean_ctor_set(x_52, 1, x_58); +lean_ctor_set(x_52, 0, x_73); +x_25 = x_52; +goto block_43; +} +else +{ +lean_object* x_74; +lean_free_object(x_52); +lean_inc(x_61); +x_74 = lean_environment_find(x_50, x_61); +if (lean_obj_tag(x_74) == 0) +{ +lean_object* x_75; lean_object* x_76; +x_75 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___closed__3; +x_76 = l_panic___at_Lean_ResolveName_resolveNamespaceUsingScope_x3f___spec__1(x_75); +x_66 = x_76; +goto block_70; +} +else +{ +uint8_t x_77; +x_77 = !lean_is_exclusive(x_74); +if (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_74, 0); +x_79 = l_Lean_ConstantInfo_type(x_78); +lean_dec(x_78); +x_80 = l_Lean_Expr_getForallBody(x_79); +lean_dec(x_79); +x_81 = l_Lean_Expr_getAppFn(x_80); +lean_dec(x_80); +if (lean_obj_tag(x_81) == 4) +{ +lean_object* x_82; +x_82 = lean_ctor_get(x_81, 0); +lean_inc(x_82); +lean_dec(x_81); +lean_ctor_set(x_74, 0, x_82); +x_66 = x_74; +goto block_70; +} +else +{ +lean_object* x_83; lean_object* x_84; +lean_dec(x_81); +lean_free_object(x_74); +x_83 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___closed__5; +x_84 = l_panic___at_Lean_ResolveName_resolveNamespaceUsingScope_x3f___spec__1(x_83); +x_66 = x_84; +goto block_70; +} +} +else +{ +lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; +x_85 = lean_ctor_get(x_74, 0); +lean_inc(x_85); +lean_dec(x_74); +x_86 = l_Lean_ConstantInfo_type(x_85); +lean_dec(x_85); +x_87 = l_Lean_Expr_getForallBody(x_86); +lean_dec(x_86); +x_88 = l_Lean_Expr_getAppFn(x_87); +lean_dec(x_87); +if (lean_obj_tag(x_88) == 4) +{ +lean_object* x_89; lean_object* x_90; +x_89 = lean_ctor_get(x_88, 0); +lean_inc(x_89); +lean_dec(x_88); +x_90 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_90, 0, x_89); +x_66 = x_90; +goto block_70; +} +else +{ +lean_object* x_91; lean_object* x_92; +lean_dec(x_88); +x_91 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___closed__5; +x_92 = l_panic___at_Lean_ResolveName_resolveNamespaceUsingScope_x3f___spec__1(x_91); +x_66 = x_92; +goto block_70; +} +} +} +} +block_70: +{ +lean_object* x_67; lean_object* x_68; lean_object* x_69; +x_67 = lean_alloc_ctor(0, 4, 1); +lean_ctor_set(x_67, 0, x_60); +lean_ctor_set(x_67, 1, x_61); +lean_ctor_set(x_67, 2, x_66); +lean_ctor_set(x_67, 3, x_65); +lean_ctor_set_uint8(x_67, sizeof(void*)*4, x_64); +x_68 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_68, 0, x_67); +if (lean_is_scalar(x_59)) { + x_69 = lean_alloc_ctor(0, 2, 0); } else { - lean_dec_ref(x_59); - x_62 = lean_box(0); + x_69 = x_59; +} +lean_ctor_set(x_69, 0, x_68); +lean_ctor_set(x_69, 1, x_58); +x_25 = x_69; +goto block_43; +} +} +else +{ +uint8_t x_93; +lean_free_object(x_52); +lean_dec(x_54); +lean_dec(x_50); +lean_dec(x_13); +x_93 = !lean_is_exclusive(x_56); +if (x_93 == 0) +{ +x_25 = x_56; +goto block_43; +} +else +{ +lean_object* x_94; lean_object* x_95; lean_object* x_96; +x_94 = lean_ctor_get(x_56, 0); +x_95 = lean_ctor_get(x_56, 1); +lean_inc(x_95); +lean_inc(x_94); +lean_dec(x_56); +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_25 = x_96; +goto block_43; +} +} +} +else +{ +lean_object* x_97; lean_object* x_98; lean_object* x_99; +x_97 = lean_ctor_get(x_52, 0); +x_98 = lean_ctor_get(x_52, 1); +lean_inc(x_98); +lean_inc(x_97); +lean_dec(x_52); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +x_99 = lean_infer_type(x_51, x_7, x_8, x_9, x_10, x_98); +if (lean_obj_tag(x_99) == 0) +{ +lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; uint8_t x_105; uint8_t x_106; uint8_t x_107; lean_object* x_108; lean_object* x_109; +x_100 = lean_ctor_get(x_99, 0); +lean_inc(x_100); +x_101 = lean_ctor_get(x_99, 1); +lean_inc(x_101); +if (lean_is_exclusive(x_99)) { + lean_ctor_release(x_99, 0); + lean_ctor_release(x_99, 1); + x_102 = x_99; +} else { + lean_dec_ref(x_99); + x_102 = lean_box(0); +} +x_103 = lean_ctor_get(x_13, 1); +lean_inc(x_103); +x_104 = lean_ctor_get(x_13, 2); +lean_inc(x_104); +lean_dec(x_13); +x_105 = 3; +x_106 = l_Lean_Elab_Command_instDecidableEqStructFieldKind(x_44, x_105); +x_107 = l_Lean_LocalDecl_binderInfo(x_97); +lean_dec(x_97); +x_108 = l_Lean_Expr_getAutoParamTactic_x3f(x_100); +lean_dec(x_100); +if (x_106 == 0) +{ +lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; +lean_dec(x_102); +lean_dec(x_50); +x_114 = lean_box(0); +x_115 = lean_alloc_ctor(0, 4, 1); +lean_ctor_set(x_115, 0, x_103); +lean_ctor_set(x_115, 1, x_104); +lean_ctor_set(x_115, 2, x_114); +lean_ctor_set(x_115, 3, x_108); +lean_ctor_set_uint8(x_115, sizeof(void*)*4, x_107); +x_116 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_116, 0, x_115); +x_117 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_117, 0, x_116); +lean_ctor_set(x_117, 1, x_101); +x_25 = x_117; +goto block_43; +} +else +{ +lean_object* x_118; +lean_inc(x_104); +x_118 = lean_environment_find(x_50, x_104); +if (lean_obj_tag(x_118) == 0) +{ +lean_object* x_119; lean_object* x_120; +x_119 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___closed__3; +x_120 = l_panic___at_Lean_ResolveName_resolveNamespaceUsingScope_x3f___spec__1(x_119); +x_109 = x_120; +goto block_113; +} +else +{ +lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; +x_121 = lean_ctor_get(x_118, 0); +lean_inc(x_121); +if (lean_is_exclusive(x_118)) { + lean_ctor_release(x_118, 0); + x_122 = x_118; +} else { + lean_dec_ref(x_118); + x_122 = lean_box(0); +} +x_123 = l_Lean_ConstantInfo_type(x_121); +lean_dec(x_121); +x_124 = l_Lean_Expr_getForallBody(x_123); +lean_dec(x_123); +x_125 = l_Lean_Expr_getAppFn(x_124); +lean_dec(x_124); +if (lean_obj_tag(x_125) == 4) +{ +lean_object* x_126; lean_object* x_127; +x_126 = lean_ctor_get(x_125, 0); +lean_inc(x_126); +lean_dec(x_125); +if (lean_is_scalar(x_122)) { + x_127 = lean_alloc_ctor(1, 1, 0); +} else { + x_127 = x_122; +} +lean_ctor_set(x_127, 0, x_126); +x_109 = x_127; +goto block_113; +} +else +{ +lean_object* x_128; lean_object* x_129; +lean_dec(x_125); +lean_dec(x_122); +x_128 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___closed__5; +x_129 = l_panic___at_Lean_ResolveName_resolveNamespaceUsingScope_x3f___spec__1(x_128); +x_109 = x_129; +goto block_113; +} +} +} +block_113: +{ +lean_object* x_110; lean_object* x_111; lean_object* x_112; +x_110 = lean_alloc_ctor(0, 4, 1); +lean_ctor_set(x_110, 0, x_103); +lean_ctor_set(x_110, 1, x_104); +lean_ctor_set(x_110, 2, x_109); +lean_ctor_set(x_110, 3, x_108); +lean_ctor_set_uint8(x_110, sizeof(void*)*4, x_107); +x_111 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_111, 0, x_110); +if (lean_is_scalar(x_102)) { + x_112 = lean_alloc_ctor(0, 2, 0); +} else { + x_112 = x_102; +} +lean_ctor_set(x_112, 0, x_111); +lean_ctor_set(x_112, 1, x_101); +x_25 = x_112; +goto block_43; +} +} +else +{ +lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; +lean_dec(x_97); +lean_dec(x_50); +lean_dec(x_13); +x_130 = lean_ctor_get(x_99, 0); +lean_inc(x_130); +x_131 = lean_ctor_get(x_99, 1); +lean_inc(x_131); +if (lean_is_exclusive(x_99)) { + lean_ctor_release(x_99, 0); + lean_ctor_release(x_99, 1); + x_132 = x_99; +} else { + lean_dec_ref(x_99); + x_132 = lean_box(0); +} +if (lean_is_scalar(x_132)) { + x_133 = lean_alloc_ctor(1, 2, 0); +} else { + x_133 = x_132; +} +lean_ctor_set(x_133, 0, x_130); +lean_ctor_set(x_133, 1, x_131); +x_25 = x_133; +goto block_43; +} +} +} +else +{ +uint8_t x_134; +lean_dec(x_51); +lean_dec(x_50); +lean_dec(x_13); +x_134 = !lean_is_exclusive(x_52); +if (x_134 == 0) +{ +x_25 = x_52; +goto block_43; +} +else +{ +lean_object* x_135; lean_object* x_136; lean_object* x_137; +x_135 = lean_ctor_get(x_52, 0); +x_136 = lean_ctor_get(x_52, 1); +lean_inc(x_136); +lean_inc(x_135); +lean_dec(x_52); +x_137 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_137, 0, x_135); +lean_ctor_set(x_137, 1, x_136); +x_25 = x_137; +goto block_43; +} +} +} +else +{ +lean_object* x_138; lean_object* x_139; +lean_dec(x_13); +x_138 = lean_box(0); +x_139 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_139, 0, x_138); +lean_ctor_set(x_139, 1, x_11); +x_25 = x_139; +goto block_43; +} +block_24: +{ +if (lean_obj_tag(x_14) == 0) +{ +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); +x_17 = 1; +x_18 = lean_usize_add(x_2, x_17); +x_2 = x_18; +x_4 = x_15; +x_11 = x_16; +goto _start; } -x_63 = 3; -x_64 = l_Lean_Elab_Command_instDecidableEqStructFieldKind(x_47, x_63); -x_65 = l_Lean_LocalDecl_binderInfo(x_57); -lean_dec(x_57); -x_66 = l_Lean_Expr_getAutoParamTactic_x3f(x_60); -lean_dec(x_60); -if (x_64 == 0) +else { -lean_object* x_72; lean_object* x_73; lean_object* x_74; -lean_dec(x_62); -lean_dec(x_54); -lean_dec(x_48); -x_72 = lean_box(0); -x_73 = lean_alloc_ctor(0, 4, 1); -lean_ctor_set(x_73, 0, x_44); -lean_ctor_set(x_73, 1, x_45); -lean_ctor_set(x_73, 2, x_72); -lean_ctor_set(x_73, 3, x_66); -lean_ctor_set_uint8(x_73, sizeof(void*)*4, x_65); -x_74 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_74, 0, x_73); -lean_ctor_set(x_55, 1, x_61); -lean_ctor_set(x_55, 0, x_74); -x_25 = x_55; -goto block_43; +uint8_t x_20; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +x_20 = !lean_is_exclusive(x_14); +if (x_20 == 0) +{ +return x_14; } else { -lean_object* x_75; -lean_free_object(x_55); -lean_inc(x_45); -x_75 = lean_environment_find(x_54, x_45); -if (lean_obj_tag(x_75) == 0) +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_14, 0); +x_22 = lean_ctor_get(x_14, 1); +lean_inc(x_22); +lean_inc(x_21); +lean_dec(x_14); +x_23 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_23, 0, x_21); +lean_ctor_set(x_23, 1, x_22); +return x_23; +} +} +} +block_43: { -lean_object* x_76; lean_object* x_77; -x_76 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___closed__3; -x_77 = l_panic___at_Lean_ResolveName_resolveNamespaceUsingScope_x3f___spec__1(x_76); -x_67 = x_77; -goto block_71; +if (lean_obj_tag(x_25) == 0) +{ +lean_object* x_26; +x_26 = lean_ctor_get(x_25, 0); +lean_inc(x_26); +if (lean_obj_tag(x_26) == 0) +{ +uint8_t x_27; +x_27 = !lean_is_exclusive(x_25); +if (x_27 == 0) +{ +lean_object* x_28; +x_28 = lean_ctor_get(x_25, 0); +lean_dec(x_28); +lean_ctor_set(x_25, 0, x_4); +x_14 = x_25; +goto block_24; } else { -uint8_t x_78; -x_78 = !lean_is_exclusive(x_75); -if (x_78 == 0) +lean_object* x_29; lean_object* x_30; +x_29 = lean_ctor_get(x_25, 1); +lean_inc(x_29); +lean_dec(x_25); +x_30 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_30, 0, x_4); +lean_ctor_set(x_30, 1, x_29); +x_14 = x_30; +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 = l_Lean_ConstantInfo_type(x_79); -lean_dec(x_79); -x_81 = l_Lean_Expr_getForallBody(x_80); -lean_dec(x_80); -x_82 = l_Lean_Expr_getAppFn(x_81); -lean_dec(x_81); -if (lean_obj_tag(x_82) == 4) +uint8_t x_31; +x_31 = !lean_is_exclusive(x_25); +if (x_31 == 0) { -lean_object* x_83; -x_83 = lean_ctor_get(x_82, 0); -lean_inc(x_83); -lean_dec(x_82); -lean_ctor_set(x_75, 0, x_83); -x_67 = x_75; -goto block_71; +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_25, 0); +lean_dec(x_32); +x_33 = lean_ctor_get(x_26, 0); +lean_inc(x_33); +lean_dec(x_26); +x_34 = lean_array_push(x_4, x_33); +lean_ctor_set(x_25, 0, x_34); +x_14 = x_25; +goto block_24; } else { -lean_object* x_84; lean_object* x_85; -lean_dec(x_82); -lean_free_object(x_75); -x_84 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___closed__5; -x_85 = l_panic___at_Lean_ResolveName_resolveNamespaceUsingScope_x3f___spec__1(x_84); -x_67 = x_85; -goto block_71; +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_35 = lean_ctor_get(x_25, 1); +lean_inc(x_35); +lean_dec(x_25); +x_36 = lean_ctor_get(x_26, 0); +lean_inc(x_36); +lean_dec(x_26); +x_37 = lean_array_push(x_4, 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_35); +x_14 = x_38; +goto block_24; +} } } else { -lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; -x_86 = lean_ctor_get(x_75, 0); -lean_inc(x_86); -lean_dec(x_75); -x_87 = l_Lean_ConstantInfo_type(x_86); -lean_dec(x_86); -x_88 = l_Lean_Expr_getForallBody(x_87); -lean_dec(x_87); -x_89 = l_Lean_Expr_getAppFn(x_88); -lean_dec(x_88); -if (lean_obj_tag(x_89) == 4) +uint8_t x_39; +lean_dec(x_4); +x_39 = !lean_is_exclusive(x_25); +if (x_39 == 0) { -lean_object* x_90; lean_object* x_91; -x_90 = lean_ctor_get(x_89, 0); -lean_inc(x_90); -lean_dec(x_89); -x_91 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_91, 0, x_90); -x_67 = x_91; -goto block_71; +x_14 = x_25; +goto block_24; } else { -lean_object* x_92; lean_object* x_93; -lean_dec(x_89); -x_92 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___closed__5; -x_93 = l_panic___at_Lean_ResolveName_resolveNamespaceUsingScope_x3f___spec__1(x_92); -x_67 = x_93; -goto block_71; +lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_40 = lean_ctor_get(x_25, 0); +x_41 = lean_ctor_get(x_25, 1); +lean_inc(x_41); +lean_inc(x_40); +lean_dec(x_25); +x_42 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_42, 0, x_40); +lean_ctor_set(x_42, 1, x_41); +x_14 = x_42; +goto block_24; } } } } -block_71: +else { -lean_object* x_68; lean_object* x_69; lean_object* x_70; -if (lean_is_scalar(x_48)) { - x_68 = lean_alloc_ctor(0, 4, 1); -} else { - x_68 = x_48; +lean_object* x_140; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +x_140 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_140, 0, x_4); +lean_ctor_set(x_140, 1, x_11); +return x_140; } -lean_ctor_set(x_68, 0, x_44); -lean_ctor_set(x_68, 1, x_45); -lean_ctor_set(x_68, 2, x_67); -lean_ctor_set(x_68, 3, x_66); -lean_ctor_set_uint8(x_68, sizeof(void*)*4, x_65); -x_69 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_69, 0, x_68); -if (lean_is_scalar(x_62)) { - x_70 = lean_alloc_ctor(0, 2, 0); -} else { - x_70 = x_62; } -lean_ctor_set(x_70, 0, x_69); -lean_ctor_set(x_70, 1, x_61); -x_25 = x_70; -goto block_43; } +LEAN_EXPORT lean_object* l_Array_filterMapM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +uint8_t x_11; +x_11 = lean_nat_dec_lt(x_2, x_3); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +x_12 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__1; +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_10); +return x_13; } else { -uint8_t x_94; -lean_free_object(x_55); -lean_dec(x_57); -lean_dec(x_54); -lean_dec(x_48); -lean_dec(x_45); -lean_dec(x_44); -x_94 = !lean_is_exclusive(x_59); -if (x_94 == 0) +lean_object* x_14; uint8_t x_15; +x_14 = lean_array_get_size(x_1); +x_15 = lean_nat_dec_le(x_3, x_14); +lean_dec(x_14); +if (x_15 == 0) { -x_25 = x_59; -goto block_43; +lean_object* x_16; lean_object* x_17; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +x_16 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___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_10); +return x_17; } else { -lean_object* x_95; lean_object* x_96; lean_object* x_97; -x_95 = lean_ctor_get(x_59, 0); -x_96 = lean_ctor_get(x_59, 1); -lean_inc(x_96); -lean_inc(x_95); -lean_dec(x_59); -x_97 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_97, 0, x_95); -lean_ctor_set(x_97, 1, x_96); -x_25 = x_97; -goto block_43; +size_t x_18; size_t x_19; lean_object* x_20; lean_object* x_21; +x_18 = lean_usize_of_nat(x_2); +x_19 = lean_usize_of_nat(x_3); +x_20 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__1; +x_21 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2(x_1, x_18, x_19, x_20, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_21; } } } -else +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure(lean_object* x_1, lean_object* x_2, lean_object* x_3, 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_98; lean_object* x_99; lean_object* x_100; -x_98 = lean_ctor_get(x_55, 0); -x_99 = lean_ctor_get(x_55, 1); -lean_inc(x_99); -lean_inc(x_98); -lean_dec(x_55); -lean_inc(x_10); -lean_inc(x_9); +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_array_get_size(x_2); +x_11 = lean_unsigned_to_nat(0u); lean_inc(x_8); -lean_inc(x_7); -x_100 = lean_infer_type(x_46, x_7, x_8, x_9, x_10, x_99); -if (lean_obj_tag(x_100) == 0) +lean_inc(x_6); +x_12 = l_Array_filterMapM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__1(x_2, x_11, x_10, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_10); +if (lean_obj_tag(x_12) == 0) { -lean_object* x_101; lean_object* x_102; lean_object* x_103; uint8_t x_104; uint8_t x_105; uint8_t x_106; lean_object* x_107; lean_object* x_108; -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_100); - x_103 = lean_box(0); -} -x_104 = 3; -x_105 = l_Lean_Elab_Command_instDecidableEqStructFieldKind(x_47, x_104); -x_106 = l_Lean_LocalDecl_binderInfo(x_98); -lean_dec(x_98); -x_107 = l_Lean_Expr_getAutoParamTactic_x3f(x_101); -lean_dec(x_101); -if (x_105 == 0) +lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_12, 1); +lean_inc(x_14); +lean_dec(x_12); +x_15 = lean_st_ref_take(x_8, x_14); +x_16 = !lean_is_exclusive(x_15); +if (x_16 == 0) +{ +lean_object* x_17; uint8_t x_18; +x_17 = lean_ctor_get(x_15, 0); +x_18 = !lean_is_exclusive(x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; +x_19 = lean_ctor_get(x_15, 1); +x_20 = lean_ctor_get(x_17, 0); +x_21 = lean_ctor_get(x_17, 4); +lean_dec(x_21); +lean_ctor_set(x_15, 1, x_13); +lean_ctor_set(x_15, 0, x_1); +x_22 = l_Lean_registerStructure(x_20, x_15); +x_23 = l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__1; +lean_ctor_set(x_17, 4, x_23); +lean_ctor_set(x_17, 0, x_22); +x_24 = lean_st_ref_set(x_8, x_17, x_19); +lean_dec(x_8); +x_25 = lean_ctor_get(x_24, 1); +lean_inc(x_25); +lean_dec(x_24); +x_26 = lean_st_ref_take(x_6, x_25); +x_27 = lean_ctor_get(x_26, 0); +lean_inc(x_27); +x_28 = lean_ctor_get(x_26, 1); +lean_inc(x_28); +lean_dec(x_26); +x_29 = !lean_is_exclusive(x_27); +if (x_29 == 0) +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; +x_30 = lean_ctor_get(x_27, 1); +lean_dec(x_30); +x_31 = l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__4; +lean_ctor_set(x_27, 1, x_31); +x_32 = lean_st_ref_set(x_6, x_27, x_28); +lean_dec(x_6); +x_33 = !lean_is_exclusive(x_32); +if (x_33 == 0) { -lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; -lean_dec(x_103); -lean_dec(x_54); -lean_dec(x_48); -x_113 = lean_box(0); -x_114 = lean_alloc_ctor(0, 4, 1); -lean_ctor_set(x_114, 0, x_44); -lean_ctor_set(x_114, 1, x_45); -lean_ctor_set(x_114, 2, x_113); -lean_ctor_set(x_114, 3, x_107); -lean_ctor_set_uint8(x_114, sizeof(void*)*4, x_106); -x_115 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_115, 0, 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_102); -x_25 = x_116; -goto block_43; +lean_object* x_34; lean_object* x_35; +x_34 = lean_ctor_get(x_32, 0); +lean_dec(x_34); +x_35 = lean_box(0); +lean_ctor_set(x_32, 0, x_35); +return x_32; } else { -lean_object* x_117; -lean_inc(x_45); -x_117 = lean_environment_find(x_54, x_45); -if (lean_obj_tag(x_117) == 0) -{ -lean_object* x_118; lean_object* x_119; -x_118 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___closed__3; -x_119 = l_panic___at_Lean_ResolveName_resolveNamespaceUsingScope_x3f___spec__1(x_118); -x_108 = x_119; -goto block_112; +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_32, 1); +lean_inc(x_36); +lean_dec(x_32); +x_37 = lean_box(0); +x_38 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_38, 0, x_37); +lean_ctor_set(x_38, 1, x_36); +return x_38; +} } else { -lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; -x_120 = lean_ctor_get(x_117, 0); -lean_inc(x_120); -if (lean_is_exclusive(x_117)) { - lean_ctor_release(x_117, 0); - x_121 = x_117; +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_39 = lean_ctor_get(x_27, 0); +x_40 = lean_ctor_get(x_27, 2); +x_41 = lean_ctor_get(x_27, 3); +x_42 = lean_ctor_get(x_27, 4); +lean_inc(x_42); +lean_inc(x_41); +lean_inc(x_40); +lean_inc(x_39); +lean_dec(x_27); +x_43 = l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__4; +x_44 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_44, 0, x_39); +lean_ctor_set(x_44, 1, x_43); +lean_ctor_set(x_44, 2, x_40); +lean_ctor_set(x_44, 3, x_41); +lean_ctor_set(x_44, 4, x_42); +x_45 = lean_st_ref_set(x_6, x_44, x_28); +lean_dec(x_6); +x_46 = lean_ctor_get(x_45, 1); +lean_inc(x_46); +if (lean_is_exclusive(x_45)) { + lean_ctor_release(x_45, 0); + lean_ctor_release(x_45, 1); + x_47 = x_45; } else { - lean_dec_ref(x_117); - x_121 = lean_box(0); + lean_dec_ref(x_45); + x_47 = lean_box(0); } -x_122 = l_Lean_ConstantInfo_type(x_120); -lean_dec(x_120); -x_123 = l_Lean_Expr_getForallBody(x_122); -lean_dec(x_122); -x_124 = l_Lean_Expr_getAppFn(x_123); -lean_dec(x_123); -if (lean_obj_tag(x_124) == 4) -{ -lean_object* x_125; lean_object* x_126; -x_125 = lean_ctor_get(x_124, 0); -lean_inc(x_125); -lean_dec(x_124); -if (lean_is_scalar(x_121)) { - x_126 = lean_alloc_ctor(1, 1, 0); +x_48 = lean_box(0); +if (lean_is_scalar(x_47)) { + x_49 = lean_alloc_ctor(0, 2, 0); } else { - x_126 = x_121; + x_49 = x_47; +} +lean_ctor_set(x_49, 0, x_48); +lean_ctor_set(x_49, 1, x_46); +return x_49; } -lean_ctor_set(x_126, 0, x_125); -x_108 = x_126; -goto block_112; } else { -lean_object* x_127; lean_object* x_128; -lean_dec(x_124); -lean_dec(x_121); -x_127 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___closed__5; -x_128 = l_panic___at_Lean_ResolveName_resolveNamespaceUsingScope_x3f___spec__1(x_127); -x_108 = x_128; -goto block_112; -} +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_50 = lean_ctor_get(x_15, 1); +x_51 = lean_ctor_get(x_17, 0); +x_52 = lean_ctor_get(x_17, 1); +x_53 = lean_ctor_get(x_17, 2); +x_54 = lean_ctor_get(x_17, 3); +x_55 = lean_ctor_get(x_17, 5); +x_56 = lean_ctor_get(x_17, 6); +lean_inc(x_56); +lean_inc(x_55); +lean_inc(x_54); +lean_inc(x_53); +lean_inc(x_52); +lean_inc(x_51); +lean_dec(x_17); +lean_ctor_set(x_15, 1, x_13); +lean_ctor_set(x_15, 0, x_1); +x_57 = l_Lean_registerStructure(x_51, x_15); +x_58 = l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__1; +x_59 = lean_alloc_ctor(0, 7, 0); +lean_ctor_set(x_59, 0, x_57); +lean_ctor_set(x_59, 1, x_52); +lean_ctor_set(x_59, 2, x_53); +lean_ctor_set(x_59, 3, x_54); +lean_ctor_set(x_59, 4, x_58); +lean_ctor_set(x_59, 5, x_55); +lean_ctor_set(x_59, 6, x_56); +x_60 = lean_st_ref_set(x_8, x_59, x_50); +lean_dec(x_8); +x_61 = lean_ctor_get(x_60, 1); +lean_inc(x_61); +lean_dec(x_60); +x_62 = lean_st_ref_take(x_6, 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); +x_66 = lean_ctor_get(x_63, 2); +lean_inc(x_66); +x_67 = lean_ctor_get(x_63, 3); +lean_inc(x_67); +x_68 = lean_ctor_get(x_63, 4); +lean_inc(x_68); +if (lean_is_exclusive(x_63)) { + lean_ctor_release(x_63, 0); + lean_ctor_release(x_63, 1); + lean_ctor_release(x_63, 2); + lean_ctor_release(x_63, 3); + lean_ctor_release(x_63, 4); + x_69 = x_63; +} else { + lean_dec_ref(x_63); + x_69 = lean_box(0); } +x_70 = l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__4; +if (lean_is_scalar(x_69)) { + x_71 = lean_alloc_ctor(0, 5, 0); +} else { + x_71 = x_69; } -block_112: -{ -lean_object* x_109; lean_object* x_110; lean_object* x_111; -if (lean_is_scalar(x_48)) { - x_109 = lean_alloc_ctor(0, 4, 1); +lean_ctor_set(x_71, 0, x_65); +lean_ctor_set(x_71, 1, x_70); +lean_ctor_set(x_71, 2, x_66); +lean_ctor_set(x_71, 3, x_67); +lean_ctor_set(x_71, 4, x_68); +x_72 = lean_st_ref_set(x_6, x_71, x_64); +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 { - x_109 = x_48; + lean_dec_ref(x_72); + x_74 = lean_box(0); } -lean_ctor_set(x_109, 0, x_44); -lean_ctor_set(x_109, 1, x_45); -lean_ctor_set(x_109, 2, x_108); -lean_ctor_set(x_109, 3, x_107); -lean_ctor_set_uint8(x_109, sizeof(void*)*4, x_106); -x_110 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_110, 0, x_109); -if (lean_is_scalar(x_103)) { - x_111 = lean_alloc_ctor(0, 2, 0); +x_75 = lean_box(0); +if (lean_is_scalar(x_74)) { + x_76 = lean_alloc_ctor(0, 2, 0); } else { - x_111 = x_103; + x_76 = x_74; } -lean_ctor_set(x_111, 0, x_110); -lean_ctor_set(x_111, 1, x_102); -x_25 = x_111; -goto block_43; +lean_ctor_set(x_76, 0, x_75); +lean_ctor_set(x_76, 1, x_73); +return x_76; } } else { -lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; -lean_dec(x_98); -lean_dec(x_54); -lean_dec(x_48); -lean_dec(x_45); -lean_dec(x_44); -x_129 = lean_ctor_get(x_100, 0); -lean_inc(x_129); -x_130 = lean_ctor_get(x_100, 1); -lean_inc(x_130); -if (lean_is_exclusive(x_100)) { - lean_ctor_release(x_100, 0); - lean_ctor_release(x_100, 1); - x_131 = x_100; +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; +x_77 = lean_ctor_get(x_15, 0); +x_78 = lean_ctor_get(x_15, 1); +lean_inc(x_78); +lean_inc(x_77); +lean_dec(x_15); +x_79 = lean_ctor_get(x_77, 0); +lean_inc(x_79); +x_80 = lean_ctor_get(x_77, 1); +lean_inc(x_80); +x_81 = lean_ctor_get(x_77, 2); +lean_inc(x_81); +x_82 = lean_ctor_get(x_77, 3); +lean_inc(x_82); +x_83 = lean_ctor_get(x_77, 5); +lean_inc(x_83); +x_84 = lean_ctor_get(x_77, 6); +lean_inc(x_84); +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); + lean_ctor_release(x_77, 6); + x_85 = x_77; } else { - lean_dec_ref(x_100); - x_131 = lean_box(0); + lean_dec_ref(x_77); + x_85 = lean_box(0); } -if (lean_is_scalar(x_131)) { - x_132 = lean_alloc_ctor(1, 2, 0); +x_86 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_86, 0, x_1); +lean_ctor_set(x_86, 1, x_13); +x_87 = l_Lean_registerStructure(x_79, x_86); +x_88 = l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__1; +if (lean_is_scalar(x_85)) { + x_89 = lean_alloc_ctor(0, 7, 0); } else { - x_132 = x_131; -} -lean_ctor_set(x_132, 0, x_129); -lean_ctor_set(x_132, 1, x_130); -x_25 = x_132; -goto block_43; -} -} + x_89 = x_85; } -else -{ -uint8_t x_133; -lean_dec(x_54); -lean_dec(x_48); -lean_dec(x_46); -lean_dec(x_45); -lean_dec(x_44); -x_133 = !lean_is_exclusive(x_55); -if (x_133 == 0) -{ -x_25 = x_55; -goto block_43; +lean_ctor_set(x_89, 0, x_87); +lean_ctor_set(x_89, 1, x_80); +lean_ctor_set(x_89, 2, x_81); +lean_ctor_set(x_89, 3, x_82); +lean_ctor_set(x_89, 4, x_88); +lean_ctor_set(x_89, 5, x_83); +lean_ctor_set(x_89, 6, x_84); +x_90 = lean_st_ref_set(x_8, x_89, x_78); +lean_dec(x_8); +x_91 = lean_ctor_get(x_90, 1); +lean_inc(x_91); +lean_dec(x_90); +x_92 = lean_st_ref_take(x_6, x_91); +x_93 = lean_ctor_get(x_92, 0); +lean_inc(x_93); +x_94 = lean_ctor_get(x_92, 1); +lean_inc(x_94); +lean_dec(x_92); +x_95 = lean_ctor_get(x_93, 0); +lean_inc(x_95); +x_96 = lean_ctor_get(x_93, 2); +lean_inc(x_96); +x_97 = lean_ctor_get(x_93, 3); +lean_inc(x_97); +x_98 = lean_ctor_get(x_93, 4); +lean_inc(x_98); +if (lean_is_exclusive(x_93)) { + lean_ctor_release(x_93, 0); + lean_ctor_release(x_93, 1); + lean_ctor_release(x_93, 2); + lean_ctor_release(x_93, 3); + lean_ctor_release(x_93, 4); + x_99 = x_93; +} else { + lean_dec_ref(x_93); + x_99 = lean_box(0); } -else -{ -lean_object* x_134; lean_object* x_135; lean_object* x_136; -x_134 = lean_ctor_get(x_55, 0); -x_135 = lean_ctor_get(x_55, 1); -lean_inc(x_135); -lean_inc(x_134); -lean_dec(x_55); -x_136 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_136, 0, x_134); -lean_ctor_set(x_136, 1, x_135); -x_25 = x_136; -goto block_43; +x_100 = l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__4; +if (lean_is_scalar(x_99)) { + x_101 = lean_alloc_ctor(0, 5, 0); +} else { + x_101 = x_99; } +lean_ctor_set(x_101, 0, x_95); +lean_ctor_set(x_101, 1, x_100); +lean_ctor_set(x_101, 2, x_96); +lean_ctor_set(x_101, 3, x_97); +lean_ctor_set(x_101, 4, x_98); +x_102 = lean_st_ref_set(x_6, x_101, x_94); +lean_dec(x_6); +x_103 = lean_ctor_get(x_102, 1); +lean_inc(x_103); +if (lean_is_exclusive(x_102)) { + lean_ctor_release(x_102, 0); + lean_ctor_release(x_102, 1); + x_104 = x_102; +} else { + lean_dec_ref(x_102); + x_104 = lean_box(0); } +x_105 = lean_box(0); +if (lean_is_scalar(x_104)) { + x_106 = lean_alloc_ctor(0, 2, 0); +} else { + x_106 = x_104; } -else -{ -lean_object* x_137; lean_object* x_138; -lean_dec(x_48); -lean_dec(x_46); -lean_dec(x_45); -lean_dec(x_44); -x_137 = lean_box(0); -x_138 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_138, 0, x_137); -lean_ctor_set(x_138, 1, x_11); -x_25 = x_138; -goto block_43; +lean_ctor_set(x_106, 0, x_105); +lean_ctor_set(x_106, 1, x_103); +return x_106; } -block_24: -{ -if (lean_obj_tag(x_14) == 0) -{ -lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; -x_15 = lean_ctor_get(x_14, 0); -lean_inc(x_15); -x_16 = lean_ctor_get(x_14, 1); -lean_inc(x_16); -lean_dec(x_14); -x_17 = 1; -x_18 = lean_usize_add(x_2, x_17); -x_2 = x_18; -x_4 = x_15; -x_11 = x_16; -goto _start; } else { -uint8_t x_20; -lean_dec(x_10); -lean_dec(x_9); +uint8_t x_107; lean_dec(x_8); -lean_dec(x_7); -x_20 = !lean_is_exclusive(x_14); -if (x_20 == 0) +lean_dec(x_6); +lean_dec(x_1); +x_107 = !lean_is_exclusive(x_12); +if (x_107 == 0) { -return x_14; +return x_12; } else { -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_14, 0); -x_22 = lean_ctor_get(x_14, 1); -lean_inc(x_22); -lean_inc(x_21); -lean_dec(x_14); -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_108; lean_object* x_109; lean_object* x_110; +x_108 = lean_ctor_get(x_12, 0); +x_109 = lean_ctor_get(x_12, 1); +lean_inc(x_109); +lean_inc(x_108); +lean_dec(x_12); +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; } } } -block_43: -{ -if (lean_obj_tag(x_25) == 0) -{ -lean_object* x_26; -x_26 = lean_ctor_get(x_25, 0); -lean_inc(x_26); -if (lean_obj_tag(x_26) == 0) -{ -uint8_t x_27; -x_27 = !lean_is_exclusive(x_25); -if (x_27 == 0) -{ -lean_object* x_28; -x_28 = lean_ctor_get(x_25, 0); -lean_dec(x_28); -lean_ctor_set(x_25, 0, x_4); -x_14 = x_25; -goto block_24; } -else +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___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_29; lean_object* x_30; -x_29 = lean_ctor_get(x_25, 1); -lean_inc(x_29); -lean_dec(x_25); -x_30 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_30, 0, x_4); -lean_ctor_set(x_30, 1, x_29); -x_14 = x_30; -goto block_24; -} +size_t x_12; size_t x_13; lean_object* x_14; +x_12 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_13 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_14 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___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_6); +lean_dec(x_5); +lean_dec(x_1); +return x_14; } -else -{ -uint8_t x_31; -x_31 = !lean_is_exclusive(x_25); -if (x_31 == 0) -{ -lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_32 = lean_ctor_get(x_25, 0); -lean_dec(x_32); -x_33 = lean_ctor_get(x_26, 0); -lean_inc(x_33); -lean_dec(x_26); -x_34 = lean_array_push(x_4, x_33); -lean_ctor_set(x_25, 0, x_34); -x_14 = x_25; -goto block_24; } -else +LEAN_EXPORT lean_object* l_Array_filterMapM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___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_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_35 = lean_ctor_get(x_25, 1); -lean_inc(x_35); -lean_dec(x_25); -x_36 = lean_ctor_get(x_26, 0); -lean_inc(x_36); -lean_dec(x_26); -x_37 = lean_array_push(x_4, 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_35); -x_14 = x_38; -goto block_24; -} +lean_object* x_11; +x_11 = l_Array_filterMapM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___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_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_11; } } -else +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, 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_39; +lean_object* x_10; +x_10 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_4); -x_39 = !lean_is_exclusive(x_25); -if (x_39 == 0) -{ -x_14 = x_25; -goto block_24; -} -else -{ -lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_40 = lean_ctor_get(x_25, 0); -x_41 = lean_ctor_get(x_25, 1); -lean_inc(x_41); -lean_inc(x_40); -lean_dec(x_25); -x_42 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_42, 0, x_40); -lean_ctor_set(x_42, 1, x_41); -x_14 = x_42; -goto block_24; -} -} +lean_dec(x_3); +lean_dec(x_2); +return x_10; } } -else +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___lambda__1(uint8_t x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: { -lean_object* x_139; +if (x_1 == 0) +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_7); -x_139 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_139, 0, x_4); -lean_ctor_set(x_139, 1, x_11); -return x_139; -} -} +lean_dec(x_4); +x_13 = lean_box(0); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_13); +lean_ctor_set(x_14, 1, x_12); +return x_14; } -LEAN_EXPORT lean_object* l_Array_filterMapM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___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: +else { -uint8_t x_11; -x_11 = lean_nat_dec_lt(x_2, x_3); -if (x_11 == 0) +if (x_2 == 0) { -lean_object* x_12; lean_object* x_13; +lean_object* x_15; lean_object* x_16; +lean_dec(x_11); +lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -x_12 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_12); -lean_ctor_set(x_13, 1, x_10); -return x_13; +lean_dec(x_4); +x_15 = lean_box(0); +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_16, 1, x_12); +return x_16; } else { -lean_object* x_14; uint8_t x_15; -x_14 = lean_array_get_size(x_1); -x_15 = lean_nat_dec_le(x_3, x_14); -lean_dec(x_14); -if (x_15 == 0) +if (x_3 == 0) { -lean_object* x_16; lean_object* x_17; +lean_object* x_17; lean_object* x_18; +lean_dec(x_11); +lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -x_16 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___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_10); -return x_17; +lean_dec(x_8); +lean_dec(x_4); +x_17 = lean_box(0); +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set(x_18, 1, x_12); +return x_18; } else { -size_t x_18; size_t x_19; lean_object* x_20; lean_object* x_21; -x_18 = lean_usize_of_nat(x_2); -x_19 = lean_usize_of_nat(x_3); -x_20 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; -x_21 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2(x_1, x_18, x_19, x_20, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_21; +lean_object* x_19; +x_19 = l_Lean_mkNoConfusion(x_4, x_8, x_9, x_10, x_11, x_12); +return x_19; } } } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure(lean_object* x_1, lean_object* x_2, lean_object* x_3, 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_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___closed__1() { _start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_10 = lean_array_get_size(x_2); -x_11 = lean_unsigned_to_nat(0u); -lean_inc(x_8); -lean_inc(x_6); -x_12 = l_Array_filterMapM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__1(x_2, x_11, x_10, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_10); -if (lean_obj_tag(x_12) == 0) -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; -x_13 = lean_ctor_get(x_12, 0); -lean_inc(x_13); -x_14 = lean_ctor_get(x_12, 1); -lean_inc(x_14); -lean_dec(x_12); -x_15 = lean_st_ref_take(x_8, x_14); -x_16 = !lean_is_exclusive(x_15); -if (x_16 == 0) -{ -lean_object* x_17; uint8_t x_18; -x_17 = lean_ctor_get(x_15, 0); -x_18 = !lean_is_exclusive(x_17); -if (x_18 == 0) -{ -lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; -x_19 = lean_ctor_get(x_15, 1); -x_20 = lean_ctor_get(x_17, 0); -x_21 = lean_ctor_get(x_17, 4); -lean_dec(x_21); -lean_ctor_set(x_15, 1, x_13); -lean_ctor_set(x_15, 0, x_1); -x_22 = l_Lean_registerStructure(x_20, x_15); -x_23 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__4; -lean_ctor_set(x_17, 4, x_23); -lean_ctor_set(x_17, 0, x_22); -x_24 = lean_st_ref_set(x_8, x_17, x_19); -lean_dec(x_8); -x_25 = lean_ctor_get(x_24, 1); -lean_inc(x_25); -lean_dec(x_24); -x_26 = lean_st_ref_take(x_6, x_25); -x_27 = lean_ctor_get(x_26, 0); -lean_inc(x_27); -x_28 = lean_ctor_get(x_26, 1); -lean_inc(x_28); -lean_dec(x_26); -x_29 = !lean_is_exclusive(x_27); -if (x_29 == 0) +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Eq", 2, 2); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___closed__2() { +_start: { -lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; -x_30 = lean_ctor_get(x_27, 1); -lean_dec(x_30); -x_31 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__7; -lean_ctor_set(x_27, 1, x_31); -x_32 = lean_st_ref_set(x_6, x_27, x_28); -lean_dec(x_6); -x_33 = !lean_is_exclusive(x_32); -if (x_33 == 0) +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___closed__3() { +_start: { -lean_object* x_34; lean_object* x_35; -x_34 = lean_ctor_get(x_32, 0); -lean_dec(x_34); -x_35 = lean_box(0); -lean_ctor_set(x_32, 0, x_35); -return x_32; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("HEq", 3, 3); +return x_1; } -else +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___closed__4() { +_start: { -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_32, 1); -lean_inc(x_36); -lean_dec(x_32); -x_37 = lean_box(0); -x_38 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_38, 0, x_37); -lean_ctor_set(x_38, 1, x_36); -return x_38; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___closed__3; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -else +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___closed__5() { +_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_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_39 = lean_ctor_get(x_27, 0); -x_40 = lean_ctor_get(x_27, 2); -x_41 = lean_ctor_get(x_27, 3); -x_42 = lean_ctor_get(x_27, 4); -lean_inc(x_42); -lean_inc(x_41); -lean_inc(x_40); -lean_inc(x_39); -lean_dec(x_27); -x_43 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__7; -x_44 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_44, 0, x_39); -lean_ctor_set(x_44, 1, x_43); -lean_ctor_set(x_44, 2, x_40); -lean_ctor_set(x_44, 3, x_41); -lean_ctor_set(x_44, 4, x_42); -x_45 = lean_st_ref_set(x_6, x_44, x_28); -lean_dec(x_6); -x_46 = lean_ctor_get(x_45, 1); -lean_inc(x_46); -if (lean_is_exclusive(x_45)) { - lean_ctor_release(x_45, 0); - lean_ctor_release(x_45, 1); - x_47 = x_45; -} else { - lean_dec_ref(x_45); - x_47 = lean_box(0); +lean_object* x_1; +x_1 = lean_mk_string_unchecked("PUnit", 5, 5); +return x_1; } -x_48 = lean_box(0); -if (lean_is_scalar(x_47)) { - x_49 = lean_alloc_ctor(0, 2, 0); -} else { - x_49 = x_47; } -lean_ctor_set(x_49, 0, x_48); -lean_ctor_set(x_49, 1, x_46); -return x_49; +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___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_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___closed__5; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -else +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions(lean_object* x_1, lean_object* x_2, lean_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_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_50 = lean_ctor_get(x_15, 1); -x_51 = lean_ctor_get(x_17, 0); -x_52 = lean_ctor_get(x_17, 1); -x_53 = lean_ctor_get(x_17, 2); -x_54 = lean_ctor_get(x_17, 3); -x_55 = lean_ctor_get(x_17, 5); -x_56 = lean_ctor_get(x_17, 6); -lean_inc(x_56); -lean_inc(x_55); -lean_inc(x_54); -lean_inc(x_53); -lean_inc(x_52); -lean_inc(x_51); -lean_dec(x_17); -lean_ctor_set(x_15, 1, x_13); -lean_ctor_set(x_15, 0, x_1); -x_57 = l_Lean_registerStructure(x_51, x_15); -x_58 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__4; -x_59 = lean_alloc_ctor(0, 7, 0); -lean_ctor_set(x_59, 0, x_57); -lean_ctor_set(x_59, 1, x_52); -lean_ctor_set(x_59, 2, x_53); -lean_ctor_set(x_59, 3, x_54); -lean_ctor_set(x_59, 4, x_58); -lean_ctor_set(x_59, 5, x_55); -lean_ctor_set(x_59, 6, x_56); -x_60 = lean_st_ref_set(x_8, x_59, x_50); -lean_dec(x_8); -x_61 = lean_ctor_get(x_60, 1); -lean_inc(x_61); -lean_dec(x_60); -x_62 = lean_st_ref_take(x_6, 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); -x_66 = lean_ctor_get(x_63, 2); -lean_inc(x_66); -x_67 = lean_ctor_get(x_63, 3); -lean_inc(x_67); -x_68 = lean_ctor_get(x_63, 4); -lean_inc(x_68); -if (lean_is_exclusive(x_63)) { - lean_ctor_release(x_63, 0); - lean_ctor_release(x_63, 1); - lean_ctor_release(x_63, 2); - lean_ctor_release(x_63, 3); - lean_ctor_release(x_63, 4); - x_69 = x_63; -} else { - lean_dec_ref(x_63); - x_69 = lean_box(0); +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; lean_object* x_15; uint8_t x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; +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, 0); +lean_inc(x_12); +lean_dec(x_10); +x_13 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___closed__2; +lean_inc(x_12); +x_14 = l_Lean_Environment_contains(x_12, x_13); +x_15 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___closed__4; +lean_inc(x_12); +x_16 = l_Lean_Environment_contains(x_12, x_15); +x_17 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___closed__6; +x_18 = l_Lean_Environment_contains(x_12, x_17); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_1); +x_19 = l_mkRecOn(x_1, x_4, x_5, x_6, x_7, x_11); +if (lean_obj_tag(x_19) == 0) +{ +if (x_18 == 0) +{ +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 = lean_box(0); +x_22 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___lambda__1(x_18, x_14, x_16, x_1, x_21, x_2, x_3, x_4, x_5, x_6, x_7, x_20); +return x_22; } -x_70 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__7; -if (lean_is_scalar(x_69)) { - x_71 = lean_alloc_ctor(0, 5, 0); -} else { - x_71 = x_69; +else +{ +lean_object* x_23; lean_object* x_24; +x_23 = lean_ctor_get(x_19, 1); +lean_inc(x_23); +lean_dec(x_19); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_1); +x_24 = l_Lean_mkCasesOn(x_1, x_4, x_5, x_6, x_7, 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_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___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___lambda__1(x_18, x_14, x_16, x_1, x_25, x_2, x_3, x_4, x_5, x_6, x_7, x_26); +lean_dec(x_25); +return x_27; } -lean_ctor_set(x_71, 0, x_65); -lean_ctor_set(x_71, 1, x_70); -lean_ctor_set(x_71, 2, x_66); -lean_ctor_set(x_71, 3, x_67); -lean_ctor_set(x_71, 4, x_68); -x_72 = lean_st_ref_set(x_6, x_71, x_64); +else +{ +uint8_t x_28; +lean_dec(x_7); 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_72); - x_74 = lean_box(0); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_1); +x_28 = !lean_is_exclusive(x_24); +if (x_28 == 0) +{ +return x_24; +} +else +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_24, 0); +x_30 = lean_ctor_get(x_24, 1); +lean_inc(x_30); +lean_inc(x_29); +lean_dec(x_24); +x_31 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_31, 0, x_29); +lean_ctor_set(x_31, 1, x_30); +return x_31; } -x_75 = lean_box(0); -if (lean_is_scalar(x_74)) { - x_76 = lean_alloc_ctor(0, 2, 0); -} else { - x_76 = x_74; } -lean_ctor_set(x_76, 0, x_75); -lean_ctor_set(x_76, 1, x_73); -return x_76; } } else { -lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; 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; -x_77 = lean_ctor_get(x_15, 0); -x_78 = lean_ctor_get(x_15, 1); -lean_inc(x_78); -lean_inc(x_77); -lean_dec(x_15); -x_79 = lean_ctor_get(x_77, 0); -lean_inc(x_79); -x_80 = lean_ctor_get(x_77, 1); -lean_inc(x_80); -x_81 = lean_ctor_get(x_77, 2); -lean_inc(x_81); -x_82 = lean_ctor_get(x_77, 3); -lean_inc(x_82); -x_83 = lean_ctor_get(x_77, 5); -lean_inc(x_83); -x_84 = lean_ctor_get(x_77, 6); -lean_inc(x_84); -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); - lean_ctor_release(x_77, 6); - x_85 = x_77; -} else { - lean_dec_ref(x_77); - x_85 = lean_box(0); +uint8_t x_32; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_1); +x_32 = !lean_is_exclusive(x_19); +if (x_32 == 0) +{ +return x_19; } -x_86 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_86, 0, x_1); -lean_ctor_set(x_86, 1, x_13); -x_87 = l_Lean_registerStructure(x_79, x_86); -x_88 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__4; -if (lean_is_scalar(x_85)) { - x_89 = lean_alloc_ctor(0, 7, 0); -} else { - x_89 = x_85; +else +{ +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_19, 0); +x_34 = lean_ctor_get(x_19, 1); +lean_inc(x_34); +lean_inc(x_33); +lean_dec(x_19); +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +return x_35; } -lean_ctor_set(x_89, 0, x_87); -lean_ctor_set(x_89, 1, x_80); -lean_ctor_set(x_89, 2, x_81); -lean_ctor_set(x_89, 3, x_82); -lean_ctor_set(x_89, 4, x_88); -lean_ctor_set(x_89, 5, x_83); -lean_ctor_set(x_89, 6, x_84); -x_90 = lean_st_ref_set(x_8, x_89, x_78); -lean_dec(x_8); -x_91 = lean_ctor_get(x_90, 1); -lean_inc(x_91); -lean_dec(x_90); -x_92 = lean_st_ref_take(x_6, x_91); -x_93 = lean_ctor_get(x_92, 0); -lean_inc(x_93); -x_94 = lean_ctor_get(x_92, 1); -lean_inc(x_94); -lean_dec(x_92); -x_95 = lean_ctor_get(x_93, 0); -lean_inc(x_95); -x_96 = lean_ctor_get(x_93, 2); -lean_inc(x_96); -x_97 = lean_ctor_get(x_93, 3); -lean_inc(x_97); -x_98 = lean_ctor_get(x_93, 4); -lean_inc(x_98); -if (lean_is_exclusive(x_93)) { - lean_ctor_release(x_93, 0); - lean_ctor_release(x_93, 1); - lean_ctor_release(x_93, 2); - lean_ctor_release(x_93, 3); - lean_ctor_release(x_93, 4); - x_99 = x_93; -} else { - lean_dec_ref(x_93); - x_99 = lean_box(0); } -x_100 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__7; -if (lean_is_scalar(x_99)) { - x_101 = lean_alloc_ctor(0, 5, 0); -} else { - x_101 = x_99; } -lean_ctor_set(x_101, 0, x_95); -lean_ctor_set(x_101, 1, x_100); -lean_ctor_set(x_101, 2, x_96); -lean_ctor_set(x_101, 3, x_97); -lean_ctor_set(x_101, 4, x_98); -x_102 = lean_st_ref_set(x_6, x_101, x_94); +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, 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; uint8_t x_15; lean_object* x_16; +x_13 = lean_unbox(x_1); +lean_dec(x_1); +x_14 = lean_unbox(x_2); +lean_dec(x_2); +x_15 = lean_unbox(x_3); +lean_dec(x_3); +x_16 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___lambda__1(x_13, x_14, x_15, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_7); lean_dec(x_6); -x_103 = lean_ctor_get(x_102, 1); -lean_inc(x_103); -if (lean_is_exclusive(x_102)) { - lean_ctor_release(x_102, 0); - lean_ctor_release(x_102, 1); - x_104 = x_102; -} else { - lean_dec_ref(x_102); - x_104 = lean_box(0); +lean_dec(x_5); +return x_16; } -x_105 = lean_box(0); -if (lean_is_scalar(x_104)) { - x_106 = lean_alloc_ctor(0, 2, 0); -} else { - x_106 = x_104; } -lean_ctor_set(x_106, 0, x_105); -lean_ctor_set(x_106, 1, x_103); -return x_106; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___boxed(lean_object* x_1, lean_object* x_2, lean_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_Structure_0__Lean_Elab_Command_mkAuxConstructions(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_3); +lean_dec(x_2); +return x_9; } } +LEAN_EXPORT lean_object* l_Lean_setReducibilityStatus___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___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) { +_start: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_10 = lean_st_ref_take(x_8, x_9); +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_10, 1); +lean_inc(x_12); +lean_dec(x_10); +x_13 = !lean_is_exclusive(x_11); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; uint8_t x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; +x_14 = lean_ctor_get(x_11, 0); +x_15 = lean_ctor_get(x_11, 4); +lean_dec(x_15); +x_16 = 0; +x_17 = lean_box(0); +x_18 = l___private_Lean_ReducibilityAttrs_0__Lean_setReducibilityStatusCore(x_14, x_1, x_2, x_16, x_17); +x_19 = l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__1; +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_take(x_6, 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; lean_object* x_28; uint8_t x_29; +x_26 = lean_ctor_get(x_23, 1); +lean_dec(x_26); +x_27 = l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__4; +lean_ctor_set(x_23, 1, x_27); +x_28 = lean_st_ref_set(x_6, x_23, x_24); +x_29 = !lean_is_exclusive(x_28); +if (x_29 == 0) +{ +lean_object* x_30; lean_object* x_31; +x_30 = lean_ctor_get(x_28, 0); +lean_dec(x_30); +x_31 = lean_box(0); +lean_ctor_set(x_28, 0, x_31); +return x_28; +} else { -uint8_t x_107; -lean_dec(x_8); -lean_dec(x_6); -lean_dec(x_1); -x_107 = !lean_is_exclusive(x_12); -if (x_107 == 0) -{ -return x_12; +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_28, 1); +lean_inc(x_32); +lean_dec(x_28); +x_33 = lean_box(0); +x_34 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_34, 0, x_33); +lean_ctor_set(x_34, 1, x_32); +return x_34; +} } else { -lean_object* x_108; lean_object* x_109; lean_object* x_110; -x_108 = lean_ctor_get(x_12, 0); -x_109 = lean_ctor_get(x_12, 1); -lean_inc(x_109); -lean_inc(x_108); -lean_dec(x_12); -x_110 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_110, 0, x_108); -lean_ctor_set(x_110, 1, x_109); -return x_110; +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_35 = lean_ctor_get(x_23, 0); +x_36 = lean_ctor_get(x_23, 2); +x_37 = lean_ctor_get(x_23, 3); +x_38 = lean_ctor_get(x_23, 4); +lean_inc(x_38); +lean_inc(x_37); +lean_inc(x_36); +lean_inc(x_35); +lean_dec(x_23); +x_39 = l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__4; +x_40 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_40, 0, x_35); +lean_ctor_set(x_40, 1, x_39); +lean_ctor_set(x_40, 2, x_36); +lean_ctor_set(x_40, 3, x_37); +lean_ctor_set(x_40, 4, x_38); +x_41 = lean_st_ref_set(x_6, x_40, x_24); +x_42 = lean_ctor_get(x_41, 1); +lean_inc(x_42); +if (lean_is_exclusive(x_41)) { + lean_ctor_release(x_41, 0); + lean_ctor_release(x_41, 1); + x_43 = x_41; +} else { + lean_dec_ref(x_41); + x_43 = lean_box(0); } +x_44 = lean_box(0); +if (lean_is_scalar(x_43)) { + x_45 = lean_alloc_ctor(0, 2, 0); +} else { + x_45 = x_43; } +lean_ctor_set(x_45, 0, x_44); +lean_ctor_set(x_45, 1, x_42); +return x_45; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: +else { -size_t x_12; size_t x_13; lean_object* x_14; -x_12 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_13 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_14 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___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_6); -lean_dec(x_5); -lean_dec(x_1); -return x_14; +lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; uint8_t x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; +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); +x_51 = lean_ctor_get(x_11, 6); +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_52 = 0; +x_53 = lean_box(0); +x_54 = l___private_Lean_ReducibilityAttrs_0__Lean_setReducibilityStatusCore(x_46, x_1, x_2, x_52, x_53); +x_55 = l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__1; +x_56 = lean_alloc_ctor(0, 7, 0); +lean_ctor_set(x_56, 0, x_54); +lean_ctor_set(x_56, 1, x_47); +lean_ctor_set(x_56, 2, x_48); +lean_ctor_set(x_56, 3, x_49); +lean_ctor_set(x_56, 4, x_55); +lean_ctor_set(x_56, 5, x_50); +lean_ctor_set(x_56, 6, 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); +lean_inc(x_60); +x_61 = lean_ctor_get(x_59, 1); +lean_inc(x_61); +lean_dec(x_59); +x_62 = lean_ctor_get(x_60, 0); +lean_inc(x_62); +x_63 = lean_ctor_get(x_60, 2); +lean_inc(x_63); +x_64 = lean_ctor_get(x_60, 3); +lean_inc(x_64); +x_65 = lean_ctor_get(x_60, 4); +lean_inc(x_65); +if (lean_is_exclusive(x_60)) { + lean_ctor_release(x_60, 0); + lean_ctor_release(x_60, 1); + lean_ctor_release(x_60, 2); + lean_ctor_release(x_60, 3); + lean_ctor_release(x_60, 4); + x_66 = x_60; +} else { + lean_dec_ref(x_60); + x_66 = lean_box(0); } +x_67 = l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__4; +if (lean_is_scalar(x_66)) { + x_68 = lean_alloc_ctor(0, 5, 0); +} else { + x_68 = x_66; } -LEAN_EXPORT lean_object* l_Array_filterMapM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; -x_11 = l_Array_filterMapM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___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_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_11; +lean_ctor_set(x_68, 0, x_62); +lean_ctor_set(x_68, 1, x_67); +lean_ctor_set(x_68, 2, x_63); +lean_ctor_set(x_68, 3, x_64); +lean_ctor_set(x_68, 4, x_65); +x_69 = lean_st_ref_set(x_6, x_68, x_61); +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_69); + x_71 = lean_box(0); } +x_72 = lean_box(0); +if (lean_is_scalar(x_71)) { + x_73 = lean_alloc_ctor(0, 2, 0); +} else { + x_73 = x_71; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; -x_10 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_10; +lean_ctor_set(x_73, 0, x_72); +lean_ctor_set(x_73, 1, x_70); +return x_73; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___lambda__1(uint8_t x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___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: { -if (x_1 == 0) +lean_object* x_12; +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +x_12 = l_Lean_Meta_mkId(x_1, 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_dec(x_11); +lean_object* x_13; lean_object* x_14; uint8_t x_15; uint8_t x_16; lean_object* x_17; +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_12, 1); +lean_inc(x_14); +lean_dec(x_12); +x_15 = 1; +x_16 = 0; +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_2); +x_17 = l_Lean_Meta_mkAuxDefinition(x_2, x_3, x_13, x_15, x_16, x_7, x_8, x_9, x_10, x_14); +if (lean_obj_tag(x_17) == 0) +{ +lean_object* x_18; uint8_t x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_17, 1); +lean_inc(x_18); +lean_dec(x_17); +x_19 = 0; +x_20 = l_Lean_setReducibilityStatus___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__1(x_2, x_19, 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); -lean_dec(x_4); -x_13 = lean_box(0); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_13); -lean_ctor_set(x_14, 1, x_12); -return x_14; +lean_dec(x_7); +return x_20; } else { -if (x_2 == 0) -{ -lean_object* x_15; lean_object* x_16; -lean_dec(x_11); +uint8_t x_21; lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_4); -x_15 = lean_box(0); -x_16 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_16, 0, x_15); -lean_ctor_set(x_16, 1, x_12); -return x_16; +lean_dec(x_7); +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; +} +} } else { -if (x_3 == 0) -{ -lean_object* x_17; lean_object* x_18; -lean_dec(x_11); +uint8_t x_25; lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_4); -x_17 = lean_box(0); -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_17); -lean_ctor_set(x_18, 1, x_12); -return x_18; +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +x_25 = !lean_is_exclusive(x_12); +if (x_25 == 0) +{ +return x_12; } else { -lean_object* x_19; -x_19 = l_Lean_mkNoConfusion(x_4, x_8, x_9, x_10, x_11, x_12); -return x_19; -} +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_12, 0); +x_27 = lean_ctor_get(x_12, 1); +lean_inc(x_27); +lean_inc(x_26); +lean_dec(x_12); +x_28 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +return x_28; } } } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___closed__1() { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("PUnit", 5, 5); +x_1 = lean_mk_string_unchecked("invalid default value for field '", 33, 33); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___closed__2() { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__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_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___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_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___closed__3() { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___closed__3() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("Eq", 2, 2); +x_1 = lean_mk_string_unchecked("', it contains metavariables", 28, 28); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___closed__4() { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___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_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___closed__3; -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_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___closed__5() { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("HEq", 3, 3); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___closed__6() { -_start: +uint8_t x_12; +x_12 = lean_usize_dec_eq(x_2, x_3); +if (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_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___closed__5; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_20; +lean_dec(x_4); +x_13 = lean_array_uget(x_1, x_2); +x_20 = lean_ctor_get(x_13, 4); +lean_inc(x_20); +if (lean_obj_tag(x_20) == 0) +{ +lean_object* x_21; +lean_dec(x_13); +x_21 = lean_box(0); +x_14 = x_21; +x_15 = x_11; +goto block_19; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions(lean_object* x_1, lean_object* x_2, lean_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; uint8_t x_14; lean_object* x_15; uint8_t x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; -x_9 = lean_st_ref_get(x_7, x_8); -x_10 = lean_ctor_get(x_9, 0); +uint8_t x_22; +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; +x_23 = lean_ctor_get(x_20, 0); +x_24 = lean_ctor_get(x_13, 2); +lean_inc(x_24); +x_25 = l_Lean_mkDefaultFnOfProjFn(x_24); +x_26 = lean_ctor_get(x_13, 3); +lean_inc(x_26); 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, 0); -lean_inc(x_12); -lean_dec(x_10); -x_13 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___closed__2; -lean_inc(x_12); -x_14 = l_Lean_Environment_contains(x_12, x_13); -x_15 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___closed__4; -lean_inc(x_12); -x_16 = l_Lean_Environment_contains(x_12, x_15); -x_17 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___closed__6; -x_18 = l_Lean_Environment_contains(x_12, x_17); +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_19 = l_mkRecOn(x_1, x_4, x_5, x_6, x_7, x_11); -if (lean_obj_tag(x_19) == 0) +x_27 = lean_infer_type(x_26, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_27) == 0) { -if (x_14 == 0) +lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t 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_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_23, x_5, x_6, x_7, x_8, x_9, x_10, x_29); +x_31 = !lean_is_exclusive(x_30); +if (x_31 == 0) { -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 = lean_box(0); -x_22 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___lambda__1(x_14, x_16, x_18, x_1, x_21, x_2, x_3, x_4, x_5, x_6, x_7, x_20); -return x_22; -} -else +lean_object* x_32; lean_object* x_33; uint8_t x_34; +x_32 = lean_ctor_get(x_30, 0); +x_33 = lean_ctor_get(x_30, 1); +x_34 = l_Lean_Expr_hasExprMVar(x_32); +if (x_34 == 0) { -lean_object* x_23; lean_object* x_24; -x_23 = lean_ctor_get(x_19, 1); -lean_inc(x_23); -lean_dec(x_19); +lean_object* x_35; lean_object* x_36; +lean_free_object(x_30); +lean_free_object(x_20); +lean_dec(x_13); +x_35 = 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_1); -x_24 = l_Lean_mkCasesOn(x_1, x_4, x_5, x_6, x_7, x_23); -if (lean_obj_tag(x_24) == 0) +x_36 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___lambda__1(x_32, x_25, x_28, x_35, x_5, x_6, x_7, x_8, x_9, x_10, x_33); +if (lean_obj_tag(x_36) == 0) { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_24, 0); -lean_inc(x_25); -x_26 = lean_ctor_get(x_24, 1); -lean_inc(x_26); -lean_dec(x_24); -x_27 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___lambda__1(x_14, x_16, x_18, x_1, x_25, x_2, x_3, x_4, x_5, x_6, x_7, x_26); -lean_dec(x_25); -return x_27; +lean_object* x_37; lean_object* x_38; +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_14 = x_37; +x_15 = x_38; +goto block_19; } else { -uint8_t x_28; +uint8_t x_39; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_1); -x_28 = !lean_is_exclusive(x_24); -if (x_28 == 0) +x_39 = !lean_is_exclusive(x_36); +if (x_39 == 0) { -return x_24; +return x_36; } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_24, 0); -x_30 = lean_ctor_get(x_24, 1); -lean_inc(x_30); -lean_inc(x_29); -lean_dec(x_24); -x_31 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_31, 0, x_29); -lean_ctor_set(x_31, 1, x_30); -return x_31; -} +lean_object* x_40; lean_object* x_41; lean_object* x_42; +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, 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; -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_1); -x_32 = !lean_is_exclusive(x_19); -if (x_32 == 0) -{ -return x_19; -} -else +lean_object* x_43; uint8_t x_44; +lean_dec(x_28); +lean_dec(x_25); +lean_inc(x_32); +x_43 = l_Lean_Meta_getMVars(x_32, x_7, x_8, x_9, x_10, x_33); +x_44 = !lean_is_exclusive(x_43); +if (x_44 == 0) { -lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_33 = lean_ctor_get(x_19, 0); -x_34 = lean_ctor_get(x_19, 1); -lean_inc(x_34); -lean_inc(x_33); -lean_dec(x_19); -x_35 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_35, 0, x_33); -lean_ctor_set(x_35, 1, x_34); -return x_35; -} -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, 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_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_45 = lean_ctor_get(x_43, 0); +x_46 = lean_ctor_get(x_43, 1); +x_47 = 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_48 = l_Lean_Elab_Term_logUnassignedUsingErrorInfos(x_45, x_47, x_5, x_6, x_7, x_8, x_9, x_10, x_46); +lean_dec(x_45); +if (lean_obj_tag(x_48) == 0) { -uint8_t x_13; uint8_t x_14; uint8_t x_15; lean_object* x_16; -x_13 = lean_unbox(x_1); -lean_dec(x_1); -x_14 = lean_unbox(x_2); -lean_dec(x_2); -x_15 = lean_unbox(x_3); -lean_dec(x_3); -x_16 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___lambda__1(x_13, x_14, x_15, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_object* x_49; lean_object* x_50; lean_object* x_51; uint8_t x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; +x_49 = lean_ctor_get(x_48, 1); +lean_inc(x_49); +lean_dec(x_48); +x_50 = lean_ctor_get(x_13, 0); +lean_inc(x_50); +x_51 = lean_ctor_get(x_13, 1); +lean_inc(x_51); +lean_dec(x_13); +x_52 = 1; +x_53 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___closed__1; +x_54 = l_Lean_Name_toString(x_51, x_52, x_53); +lean_ctor_set_tag(x_20, 3); +lean_ctor_set(x_20, 0, x_54); +x_55 = l_Lean_MessageData_ofFormat(x_20); +x_56 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___closed__2; +lean_ctor_set_tag(x_43, 7); +lean_ctor_set(x_43, 1, x_55); +lean_ctor_set(x_43, 0, x_56); +x_57 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___closed__4; +lean_ctor_set_tag(x_30, 7); +lean_ctor_set(x_30, 1, x_57); +lean_ctor_set(x_30, 0, x_43); +x_58 = l_Lean_indentExpr(x_32); +x_59 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_59, 0, x_30); +lean_ctor_set(x_59, 1, x_58); +x_60 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3; +x_61 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_61, 0, x_59); +lean_ctor_set(x_61, 1, x_60); +x_62 = l_Lean_throwErrorAt___at___private_Lean_Elab_Binders_0__Lean_Elab_Term_elabBinderViews_loop___spec__1(x_50, x_61, x_5, x_6, x_7, x_8, x_9, x_10, x_49); +lean_dec(x_10); +lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -return x_16; -} +lean_dec(x_50); +x_63 = !lean_is_exclusive(x_62); +if (x_63 == 0) +{ +return x_62; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___boxed(lean_object* x_1, lean_object* x_2, lean_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___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_3); -lean_dec(x_2); -return x_9; +lean_object* 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(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_Lean_setReducibilityStatus___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___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) { -_start: +else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_10 = lean_st_ref_take(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); +uint8_t x_67; +lean_free_object(x_43); +lean_free_object(x_30); +lean_dec(x_32); +lean_free_object(x_20); +lean_dec(x_13); lean_dec(x_10); -x_13 = !lean_is_exclusive(x_11); -if (x_13 == 0) -{ -lean_object* x_14; lean_object* x_15; uint8_t x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; -x_14 = lean_ctor_get(x_11, 0); -x_15 = lean_ctor_get(x_11, 4); -lean_dec(x_15); -x_16 = 0; -x_17 = lean_box(0); -x_18 = l___private_Lean_ReducibilityAttrs_0__Lean_setReducibilityStatusCore(x_14, x_1, x_2, x_16, x_17); -x_19 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__4; -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_take(x_6, 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; lean_object* x_28; uint8_t x_29; -x_26 = lean_ctor_get(x_23, 1); -lean_dec(x_26); -x_27 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__7; -lean_ctor_set(x_23, 1, x_27); -x_28 = lean_st_ref_set(x_6, x_23, x_24); -x_29 = !lean_is_exclusive(x_28); -if (x_29 == 0) +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_67 = !lean_is_exclusive(x_48); +if (x_67 == 0) { -lean_object* x_30; lean_object* x_31; -x_30 = lean_ctor_get(x_28, 0); -lean_dec(x_30); -x_31 = lean_box(0); -lean_ctor_set(x_28, 0, x_31); -return x_28; +return x_48; } else { -lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_32 = lean_ctor_get(x_28, 1); -lean_inc(x_32); -lean_dec(x_28); -x_33 = lean_box(0); -x_34 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_34, 0, x_33); -lean_ctor_set(x_34, 1, x_32); -return x_34; +lean_object* x_68; lean_object* x_69; lean_object* x_70; +x_68 = lean_ctor_get(x_48, 0); +x_69 = lean_ctor_get(x_48, 1); +lean_inc(x_69); +lean_inc(x_68); +lean_dec(x_48); +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_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_35 = lean_ctor_get(x_23, 0); -x_36 = lean_ctor_get(x_23, 2); -x_37 = lean_ctor_get(x_23, 3); -x_38 = lean_ctor_get(x_23, 4); -lean_inc(x_38); -lean_inc(x_37); -lean_inc(x_36); -lean_inc(x_35); -lean_dec(x_23); -x_39 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__7; -x_40 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_40, 0, x_35); -lean_ctor_set(x_40, 1, x_39); -lean_ctor_set(x_40, 2, x_36); -lean_ctor_set(x_40, 3, x_37); -lean_ctor_set(x_40, 4, x_38); -x_41 = lean_st_ref_set(x_6, x_40, x_24); -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_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; +x_71 = lean_ctor_get(x_43, 0); +x_72 = lean_ctor_get(x_43, 1); +lean_inc(x_72); +lean_inc(x_71); +lean_dec(x_43); +x_73 = 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_74 = l_Lean_Elab_Term_logUnassignedUsingErrorInfos(x_71, x_73, x_5, x_6, x_7, x_8, x_9, x_10, x_72); +lean_dec(x_71); +if (lean_obj_tag(x_74) == 0) +{ +lean_object* x_75; 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; 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_75 = lean_ctor_get(x_74, 1); +lean_inc(x_75); +lean_dec(x_74); +x_76 = lean_ctor_get(x_13, 0); +lean_inc(x_76); +x_77 = lean_ctor_get(x_13, 1); +lean_inc(x_77); +lean_dec(x_13); +x_78 = 1; +x_79 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___closed__1; +x_80 = l_Lean_Name_toString(x_77, x_78, x_79); +lean_ctor_set_tag(x_20, 3); +lean_ctor_set(x_20, 0, x_80); +x_81 = l_Lean_MessageData_ofFormat(x_20); +x_82 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___closed__2; +x_83 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_83, 0, x_82); +lean_ctor_set(x_83, 1, x_81); +x_84 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___closed__4; +lean_ctor_set_tag(x_30, 7); +lean_ctor_set(x_30, 1, x_84); +lean_ctor_set(x_30, 0, x_83); +x_85 = l_Lean_indentExpr(x_32); +x_86 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_86, 0, x_30); +lean_ctor_set(x_86, 1, x_85); +x_87 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3; +x_88 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_88, 0, x_86); +lean_ctor_set(x_88, 1, x_87); +x_89 = l_Lean_throwErrorAt___at___private_Lean_Elab_Binders_0__Lean_Elab_Term_elabBinderViews_loop___spec__1(x_76, x_88, x_5, x_6, x_7, x_8, x_9, x_10, x_75); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_76); +x_90 = lean_ctor_get(x_89, 0); +lean_inc(x_90); +x_91 = lean_ctor_get(x_89, 1); +lean_inc(x_91); +if (lean_is_exclusive(x_89)) { + lean_ctor_release(x_89, 0); + lean_ctor_release(x_89, 1); + x_92 = x_89; } else { - lean_dec_ref(x_41); - x_43 = lean_box(0); + lean_dec_ref(x_89); + x_92 = lean_box(0); } -x_44 = lean_box(0); -if (lean_is_scalar(x_43)) { - x_45 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_92)) { + x_93 = lean_alloc_ctor(1, 2, 0); } else { - x_45 = x_43; -} -lean_ctor_set(x_45, 0, x_44); -lean_ctor_set(x_45, 1, x_42); -return x_45; + x_93 = x_92; } +lean_ctor_set(x_93, 0, x_90); +lean_ctor_set(x_93, 1, x_91); +return x_93; } else { -lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; uint8_t x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; -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); -x_51 = lean_ctor_get(x_11, 6); -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_52 = 0; -x_53 = lean_box(0); -x_54 = l___private_Lean_ReducibilityAttrs_0__Lean_setReducibilityStatusCore(x_46, x_1, x_2, x_52, x_53); -x_55 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__4; -x_56 = lean_alloc_ctor(0, 7, 0); -lean_ctor_set(x_56, 0, x_54); -lean_ctor_set(x_56, 1, x_47); -lean_ctor_set(x_56, 2, x_48); -lean_ctor_set(x_56, 3, x_49); -lean_ctor_set(x_56, 4, x_55); -lean_ctor_set(x_56, 5, x_50); -lean_ctor_set(x_56, 6, 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); -lean_inc(x_60); -x_61 = lean_ctor_get(x_59, 1); -lean_inc(x_61); -lean_dec(x_59); -x_62 = lean_ctor_get(x_60, 0); -lean_inc(x_62); -x_63 = lean_ctor_get(x_60, 2); -lean_inc(x_63); -x_64 = lean_ctor_get(x_60, 3); -lean_inc(x_64); -x_65 = lean_ctor_get(x_60, 4); -lean_inc(x_65); -if (lean_is_exclusive(x_60)) { - lean_ctor_release(x_60, 0); - lean_ctor_release(x_60, 1); - lean_ctor_release(x_60, 2); - lean_ctor_release(x_60, 3); - lean_ctor_release(x_60, 4); - x_66 = x_60; -} else { - lean_dec_ref(x_60); - x_66 = lean_box(0); -} -x_67 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__7; -if (lean_is_scalar(x_66)) { - x_68 = lean_alloc_ctor(0, 5, 0); +lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; +lean_free_object(x_30); +lean_dec(x_32); +lean_free_object(x_20); +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); +x_94 = lean_ctor_get(x_74, 0); +lean_inc(x_94); +x_95 = lean_ctor_get(x_74, 1); +lean_inc(x_95); +if (lean_is_exclusive(x_74)) { + lean_ctor_release(x_74, 0); + lean_ctor_release(x_74, 1); + x_96 = x_74; } else { - x_68 = x_66; + lean_dec_ref(x_74); + x_96 = lean_box(0); } -lean_ctor_set(x_68, 0, x_62); -lean_ctor_set(x_68, 1, x_67); -lean_ctor_set(x_68, 2, x_63); -lean_ctor_set(x_68, 3, x_64); -lean_ctor_set(x_68, 4, x_65); -x_69 = lean_st_ref_set(x_6, x_68, x_61); -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; +if (lean_is_scalar(x_96)) { + x_97 = lean_alloc_ctor(1, 2, 0); } else { - lean_dec_ref(x_69); - x_71 = lean_box(0); + x_97 = x_96; } -x_72 = lean_box(0); -if (lean_is_scalar(x_71)) { - x_73 = lean_alloc_ctor(0, 2, 0); -} else { - x_73 = x_71; +lean_ctor_set(x_97, 0, x_94); +lean_ctor_set(x_97, 1, x_95); +return x_97; } -lean_ctor_set(x_73, 0, x_72); -lean_ctor_set(x_73, 1, x_70); -return x_73; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___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: +else { -lean_object* x_12; -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -x_12 = l_Lean_Meta_mkId(x_1, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_12) == 0) +lean_object* x_98; lean_object* x_99; uint8_t x_100; +x_98 = lean_ctor_get(x_30, 0); +x_99 = lean_ctor_get(x_30, 1); +lean_inc(x_99); +lean_inc(x_98); +lean_dec(x_30); +x_100 = l_Lean_Expr_hasExprMVar(x_98); +if (x_100 == 0) { -lean_object* x_13; lean_object* x_14; uint8_t x_15; uint8_t x_16; lean_object* x_17; -x_13 = lean_ctor_get(x_12, 0); -lean_inc(x_13); -x_14 = lean_ctor_get(x_12, 1); -lean_inc(x_14); -lean_dec(x_12); -x_15 = 1; -x_16 = 0; +lean_object* x_101; lean_object* x_102; +lean_free_object(x_20); +lean_dec(x_13); +x_101 = lean_box(0); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_2); -x_17 = l_Lean_Meta_mkAuxDefinition(x_2, x_3, x_13, x_15, x_16, x_7, x_8, x_9, x_10, x_14); -if (lean_obj_tag(x_17) == 0) +x_102 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___lambda__1(x_98, x_25, x_28, x_101, x_5, x_6, x_7, x_8, x_9, x_10, x_99); +if (lean_obj_tag(x_102) == 0) { -lean_object* x_18; uint8_t x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_17, 1); -lean_inc(x_18); -lean_dec(x_17); -x_19 = 0; -x_20 = l_Lean_setReducibilityStatus___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__1(x_2, x_19, 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); -lean_dec(x_7); -return x_20; +lean_object* x_103; lean_object* x_104; +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_14 = x_103; +x_15 = x_104; +goto block_19; } else { -uint8_t x_21; +lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -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_dec(x_6); +lean_dec(x_5); +x_105 = lean_ctor_get(x_102, 0); +lean_inc(x_105); +x_106 = lean_ctor_get(x_102, 1); +lean_inc(x_106); +if (lean_is_exclusive(x_102)) { + lean_ctor_release(x_102, 0); + lean_ctor_release(x_102, 1); + x_107 = x_102; +} else { + lean_dec_ref(x_102); + x_107 = lean_box(0); } +if (lean_is_scalar(x_107)) { + x_108 = lean_alloc_ctor(1, 2, 0); +} else { + x_108 = x_107; } +lean_ctor_set(x_108, 0, x_105); +lean_ctor_set(x_108, 1, x_106); +return x_108; } -else -{ -uint8_t x_25; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -x_25 = !lean_is_exclusive(x_12); -if (x_25 == 0) -{ -return x_12; } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_12, 0); -x_27 = lean_ctor_get(x_12, 1); -lean_inc(x_27); -lean_inc(x_26); -lean_dec(x_12); -x_28 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_28, 0, x_26); -lean_ctor_set(x_28, 1, x_27); -return x_28; -} -} -} -} -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("invalid default value for field, it contains metavariables", 58, 58); -return x_1; -} -} -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} +lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; +lean_dec(x_28); +lean_dec(x_25); +lean_inc(x_98); +x_109 = l_Lean_Meta_getMVars(x_98, x_7, x_8, x_9, x_10, x_99); +x_110 = lean_ctor_get(x_109, 0); +lean_inc(x_110); +x_111 = lean_ctor_get(x_109, 1); +lean_inc(x_111); +if (lean_is_exclusive(x_109)) { + lean_ctor_release(x_109, 0); + lean_ctor_release(x_109, 1); + x_112 = x_109; +} else { + lean_dec_ref(x_109); + x_112 = lean_box(0); } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -uint8_t x_12; -x_12 = lean_usize_dec_eq(x_2, x_3); -if (x_12 == 0) -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; -lean_dec(x_4); -x_13 = lean_array_uget(x_1, x_2); -x_14 = lean_ctor_get(x_13, 1); -lean_inc(x_14); -x_15 = lean_ctor_get(x_13, 0); -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; uint8_t x_20; -x_17 = lean_ctor_get(x_14, 0); -x_18 = lean_ctor_get(x_14, 1); -x_19 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -x_20 = !lean_is_exclusive(x_19); -if (x_20 == 0) -{ -lean_object* x_21; lean_object* x_22; uint8_t x_23; -x_21 = lean_ctor_get(x_19, 0); -x_22 = lean_ctor_get(x_19, 1); -x_23 = l_Lean_Expr_hasExprMVar(x_21); -if (x_23 == 0) -{ -lean_object* x_24; lean_object* x_25; -lean_free_object(x_19); -lean_free_object(x_14); -x_24 = lean_box(0); +x_113 = lean_box(0); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -x_25 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___lambda__1(x_21, x_15, x_17, x_24, x_5, x_6, x_7, x_8, x_9, x_10, x_22); -if (lean_obj_tag(x_25) == 0) +lean_inc(x_6); +lean_inc(x_5); +x_114 = l_Lean_Elab_Term_logUnassignedUsingErrorInfos(x_110, x_113, x_5, x_6, x_7, x_8, x_9, x_10, x_111); +lean_dec(x_110); +if (lean_obj_tag(x_114) == 0) { -lean_object* x_26; lean_object* x_27; size_t x_28; size_t x_29; -x_26 = lean_ctor_get(x_25, 0); -lean_inc(x_26); -x_27 = lean_ctor_get(x_25, 1); -lean_inc(x_27); -lean_dec(x_25); -x_28 = 1; -x_29 = lean_usize_add(x_2, x_28); -x_2 = x_29; -x_4 = x_26; -x_11 = x_27; -goto _start; +lean_object* x_115; lean_object* x_116; lean_object* x_117; uint8_t x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_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_115 = lean_ctor_get(x_114, 1); +lean_inc(x_115); +lean_dec(x_114); +x_116 = lean_ctor_get(x_13, 0); +lean_inc(x_116); +x_117 = lean_ctor_get(x_13, 1); +lean_inc(x_117); +lean_dec(x_13); +x_118 = 1; +x_119 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___closed__1; +x_120 = l_Lean_Name_toString(x_117, x_118, x_119); +lean_ctor_set_tag(x_20, 3); +lean_ctor_set(x_20, 0, x_120); +x_121 = l_Lean_MessageData_ofFormat(x_20); +x_122 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___closed__2; +if (lean_is_scalar(x_112)) { + x_123 = lean_alloc_ctor(7, 2, 0); +} else { + x_123 = x_112; + lean_ctor_set_tag(x_123, 7); +} +lean_ctor_set(x_123, 0, x_122); +lean_ctor_set(x_123, 1, x_121); +x_124 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___closed__4; +x_125 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_125, 0, x_123); +lean_ctor_set(x_125, 1, x_124); +x_126 = l_Lean_indentExpr(x_98); +x_127 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_127, 0, x_125); +lean_ctor_set(x_127, 1, x_126); +x_128 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3; +x_129 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_129, 0, x_127); +lean_ctor_set(x_129, 1, x_128); +x_130 = l_Lean_throwErrorAt___at___private_Lean_Elab_Binders_0__Lean_Elab_Term_elabBinderViews_loop___spec__1(x_116, x_129, x_5, x_6, x_7, x_8, x_9, x_10, x_115); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_116); +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); +} +if (lean_is_scalar(x_133)) { + x_134 = lean_alloc_ctor(1, 2, 0); +} else { + x_134 = x_133; +} +lean_ctor_set(x_134, 0, x_131); +lean_ctor_set(x_134, 1, x_132); +return x_134; } else { -uint8_t x_31; +lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; +lean_dec(x_112); +lean_dec(x_98); +lean_free_object(x_20); +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); -x_31 = !lean_is_exclusive(x_25); -if (x_31 == 0) -{ -return x_25; +x_135 = lean_ctor_get(x_114, 0); +lean_inc(x_135); +x_136 = lean_ctor_get(x_114, 1); +lean_inc(x_136); +if (lean_is_exclusive(x_114)) { + lean_ctor_release(x_114, 0); + lean_ctor_release(x_114, 1); + x_137 = x_114; +} else { + lean_dec_ref(x_114); + x_137 = lean_box(0); +} +if (lean_is_scalar(x_137)) { + x_138 = lean_alloc_ctor(1, 2, 0); +} else { + x_138 = x_137; +} +lean_ctor_set(x_138, 0, x_135); +lean_ctor_set(x_138, 1, x_136); +return x_138; } -else -{ -lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_32 = lean_ctor_get(x_25, 0); -x_33 = lean_ctor_get(x_25, 1); -lean_inc(x_33); -lean_inc(x_32); -lean_dec(x_25); -x_34 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_34, 0, x_32); -lean_ctor_set(x_34, 1, x_33); -return x_34; } } } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; -lean_dec(x_17); -lean_dec(x_15); -x_35 = l_Lean_indentExpr(x_21); -x_36 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___closed__2; -lean_ctor_set_tag(x_19, 7); -lean_ctor_set(x_19, 1, x_35); -lean_ctor_set(x_19, 0, x_36); -x_37 = l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__4; -lean_ctor_set_tag(x_14, 7); -lean_ctor_set(x_14, 1, x_37); -lean_ctor_set(x_14, 0, x_19); -x_38 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_22); +uint8_t x_139; +lean_dec(x_25); +lean_free_object(x_20); +lean_dec(x_23); +lean_dec(x_13); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -x_39 = !lean_is_exclusive(x_38); -if (x_39 == 0) +lean_dec(x_6); +lean_dec(x_5); +x_139 = !lean_is_exclusive(x_27); +if (x_139 == 0) { -return x_38; +return x_27; } 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; +lean_object* x_140; lean_object* x_141; lean_object* x_142; +x_140 = lean_ctor_get(x_27, 0); +x_141 = lean_ctor_get(x_27, 1); +lean_inc(x_141); +lean_inc(x_140); +lean_dec(x_27); +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_43; lean_object* x_44; uint8_t x_45; -x_43 = lean_ctor_get(x_19, 0); -x_44 = lean_ctor_get(x_19, 1); -lean_inc(x_44); -lean_inc(x_43); -lean_dec(x_19); -x_45 = l_Lean_Expr_hasExprMVar(x_43); -if (x_45 == 0) -{ -lean_object* x_46; lean_object* x_47; -lean_free_object(x_14); -x_46 = lean_box(0); +lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; +x_143 = lean_ctor_get(x_20, 0); +lean_inc(x_143); +lean_dec(x_20); +x_144 = lean_ctor_get(x_13, 2); +lean_inc(x_144); +x_145 = l_Lean_mkDefaultFnOfProjFn(x_144); +x_146 = lean_ctor_get(x_13, 3); +lean_inc(x_146); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -x_47 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___lambda__1(x_43, x_15, x_17, x_46, x_5, x_6, x_7, x_8, x_9, x_10, x_44); -if (lean_obj_tag(x_47) == 0) -{ -lean_object* x_48; lean_object* x_49; size_t x_50; size_t x_51; -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 = 1; -x_51 = lean_usize_add(x_2, x_50); -x_2 = x_51; -x_4 = x_48; -x_11 = x_49; -goto _start; -} -else +x_147 = lean_infer_type(x_146, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_147) == 0) { -lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_5); -x_53 = lean_ctor_get(x_47, 0); -lean_inc(x_53); -x_54 = lean_ctor_get(x_47, 1); -lean_inc(x_54); -if (lean_is_exclusive(x_47)) { - lean_ctor_release(x_47, 0); - lean_ctor_release(x_47, 1); - x_55 = x_47; -} else { - lean_dec_ref(x_47); - x_55 = lean_box(0); -} -if (lean_is_scalar(x_55)) { - x_56 = lean_alloc_ctor(1, 2, 0); +lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; uint8_t x_154; +x_148 = lean_ctor_get(x_147, 0); +lean_inc(x_148); +x_149 = lean_ctor_get(x_147, 1); +lean_inc(x_149); +lean_dec(x_147); +x_150 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_143, x_5, x_6, x_7, x_8, x_9, x_10, x_149); +x_151 = lean_ctor_get(x_150, 0); +lean_inc(x_151); +x_152 = lean_ctor_get(x_150, 1); +lean_inc(x_152); +if (lean_is_exclusive(x_150)) { + lean_ctor_release(x_150, 0); + lean_ctor_release(x_150, 1); + x_153 = x_150; } else { - x_56 = x_55; -} -lean_ctor_set(x_56, 0, x_53); -lean_ctor_set(x_56, 1, x_54); -return x_56; + lean_dec_ref(x_150); + x_153 = lean_box(0); } +x_154 = l_Lean_Expr_hasExprMVar(x_151); +if (x_154 == 0) +{ +lean_object* x_155; lean_object* x_156; +lean_dec(x_153); +lean_dec(x_13); +x_155 = lean_box(0); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +x_156 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___lambda__1(x_151, x_145, x_148, x_155, x_5, x_6, x_7, x_8, x_9, x_10, x_152); +if (lean_obj_tag(x_156) == 0) +{ +lean_object* x_157; lean_object* x_158; +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_14 = x_157; +x_15 = x_158; +goto block_19; } else { -lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; -lean_dec(x_17); -lean_dec(x_15); -x_57 = l_Lean_indentExpr(x_43); -x_58 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___closed__2; -x_59 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_59, 0, x_58); -lean_ctor_set(x_59, 1, x_57); -x_60 = l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__4; -lean_ctor_set_tag(x_14, 7); -lean_ctor_set(x_14, 1, x_60); -lean_ctor_set(x_14, 0, x_59); -x_61 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_44); +lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -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_dec(x_6); +lean_dec(x_5); +x_159 = lean_ctor_get(x_156, 0); +lean_inc(x_159); +x_160 = lean_ctor_get(x_156, 1); +lean_inc(x_160); +if (lean_is_exclusive(x_156)) { + lean_ctor_release(x_156, 0); + lean_ctor_release(x_156, 1); + x_161 = x_156; } else { - lean_dec_ref(x_61); - x_64 = lean_box(0); + lean_dec_ref(x_156); + x_161 = lean_box(0); } -if (lean_is_scalar(x_64)) { - x_65 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_161)) { + x_162 = lean_alloc_ctor(1, 2, 0); } else { - x_65 = x_64; -} -lean_ctor_set(x_65, 0, x_62); -lean_ctor_set(x_65, 1, x_63); -return x_65; + x_162 = x_161; } +lean_ctor_set(x_162, 0, x_159); +lean_ctor_set(x_162, 1, x_160); +return x_162; } } else { -lean_object* x_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_66 = lean_ctor_get(x_14, 0); -x_67 = lean_ctor_get(x_14, 1); -lean_inc(x_67); -lean_inc(x_66); -lean_dec(x_14); -x_68 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_67, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -x_69 = lean_ctor_get(x_68, 0); -lean_inc(x_69); -x_70 = lean_ctor_get(x_68, 1); -lean_inc(x_70); -if (lean_is_exclusive(x_68)) { - lean_ctor_release(x_68, 0); - lean_ctor_release(x_68, 1); - x_71 = x_68; +lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; +lean_dec(x_148); +lean_dec(x_145); +lean_inc(x_151); +x_163 = l_Lean_Meta_getMVars(x_151, x_7, x_8, x_9, x_10, x_152); +x_164 = lean_ctor_get(x_163, 0); +lean_inc(x_164); +x_165 = lean_ctor_get(x_163, 1); +lean_inc(x_165); +if (lean_is_exclusive(x_163)) { + lean_ctor_release(x_163, 0); + lean_ctor_release(x_163, 1); + x_166 = x_163; } else { - lean_dec_ref(x_68); - x_71 = lean_box(0); + lean_dec_ref(x_163); + x_166 = lean_box(0); } -x_72 = l_Lean_Expr_hasExprMVar(x_69); -if (x_72 == 0) -{ -lean_object* x_73; lean_object* x_74; -lean_dec(x_71); -x_73 = lean_box(0); +x_167 = lean_box(0); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -x_74 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___lambda__1(x_69, x_15, x_66, x_73, x_5, x_6, x_7, x_8, x_9, x_10, x_70); -if (lean_obj_tag(x_74) == 0) +lean_inc(x_6); +lean_inc(x_5); +x_168 = l_Lean_Elab_Term_logUnassignedUsingErrorInfos(x_164, x_167, x_5, x_6, x_7, x_8, x_9, x_10, x_165); +lean_dec(x_164); +if (lean_obj_tag(x_168) == 0) { -lean_object* x_75; lean_object* x_76; size_t x_77; size_t x_78; -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 = 1; -x_78 = lean_usize_add(x_2, x_77); -x_2 = x_78; -x_4 = x_75; -x_11 = x_76; -goto _start; +lean_object* x_169; lean_object* x_170; lean_object* x_171; uint8_t x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; +x_169 = lean_ctor_get(x_168, 1); +lean_inc(x_169); +lean_dec(x_168); +x_170 = lean_ctor_get(x_13, 0); +lean_inc(x_170); +x_171 = lean_ctor_get(x_13, 1); +lean_inc(x_171); +lean_dec(x_13); +x_172 = 1; +x_173 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___closed__1; +x_174 = l_Lean_Name_toString(x_171, x_172, x_173); +x_175 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_175, 0, x_174); +x_176 = l_Lean_MessageData_ofFormat(x_175); +x_177 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___closed__2; +if (lean_is_scalar(x_166)) { + x_178 = lean_alloc_ctor(7, 2, 0); +} else { + x_178 = x_166; + lean_ctor_set_tag(x_178, 7); +} +lean_ctor_set(x_178, 0, x_177); +lean_ctor_set(x_178, 1, x_176); +x_179 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___closed__4; +if (lean_is_scalar(x_153)) { + x_180 = lean_alloc_ctor(7, 2, 0); +} else { + x_180 = x_153; + lean_ctor_set_tag(x_180, 7); +} +lean_ctor_set(x_180, 0, x_178); +lean_ctor_set(x_180, 1, x_179); +x_181 = l_Lean_indentExpr(x_151); +x_182 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_182, 0, x_180); +lean_ctor_set(x_182, 1, x_181); +x_183 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3; +x_184 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_184, 0, x_182); +lean_ctor_set(x_184, 1, x_183); +x_185 = l_Lean_throwErrorAt___at___private_Lean_Elab_Binders_0__Lean_Elab_Term_elabBinderViews_loop___spec__1(x_170, x_184, x_5, x_6, x_7, x_8, x_9, x_10, x_169); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_170); +x_186 = lean_ctor_get(x_185, 0); +lean_inc(x_186); +x_187 = lean_ctor_get(x_185, 1); +lean_inc(x_187); +if (lean_is_exclusive(x_185)) { + lean_ctor_release(x_185, 0); + lean_ctor_release(x_185, 1); + x_188 = x_185; +} else { + lean_dec_ref(x_185); + x_188 = lean_box(0); +} +if (lean_is_scalar(x_188)) { + x_189 = lean_alloc_ctor(1, 2, 0); +} else { + x_189 = x_188; +} +lean_ctor_set(x_189, 0, x_186); +lean_ctor_set(x_189, 1, x_187); +return x_189; } else { -lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; +lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; +lean_dec(x_166); +lean_dec(x_153); +lean_dec(x_151); +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); -x_80 = lean_ctor_get(x_74, 0); -lean_inc(x_80); -x_81 = lean_ctor_get(x_74, 1); -lean_inc(x_81); -if (lean_is_exclusive(x_74)) { - lean_ctor_release(x_74, 0); - lean_ctor_release(x_74, 1); - x_82 = x_74; +x_190 = lean_ctor_get(x_168, 0); +lean_inc(x_190); +x_191 = lean_ctor_get(x_168, 1); +lean_inc(x_191); +if (lean_is_exclusive(x_168)) { + lean_ctor_release(x_168, 0); + lean_ctor_release(x_168, 1); + x_192 = x_168; } else { - lean_dec_ref(x_74); - x_82 = lean_box(0); + lean_dec_ref(x_168); + x_192 = lean_box(0); } -if (lean_is_scalar(x_82)) { - x_83 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_192)) { + x_193 = lean_alloc_ctor(1, 2, 0); } else { - x_83 = x_82; + x_193 = x_192; +} +lean_ctor_set(x_193, 0, x_190); +lean_ctor_set(x_193, 1, x_191); +return x_193; } -lean_ctor_set(x_83, 0, x_80); -lean_ctor_set(x_83, 1, x_81); -return x_83; } } else { -lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; -lean_dec(x_66); -lean_dec(x_15); -x_84 = l_Lean_indentExpr(x_69); -x_85 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___closed__2; -if (lean_is_scalar(x_71)) { - x_86 = lean_alloc_ctor(7, 2, 0); -} else { - x_86 = x_71; - lean_ctor_set_tag(x_86, 7); -} -lean_ctor_set(x_86, 0, x_85); -lean_ctor_set(x_86, 1, x_84); -x_87 = l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__4; -x_88 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_88, 0, x_86); -lean_ctor_set(x_88, 1, x_87); -x_89 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_88, x_5, x_6, x_7, x_8, x_9, x_10, x_70); +lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; +lean_dec(x_145); +lean_dec(x_143); +lean_dec(x_13); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -x_90 = lean_ctor_get(x_89, 0); -lean_inc(x_90); -x_91 = lean_ctor_get(x_89, 1); -lean_inc(x_91); -if (lean_is_exclusive(x_89)) { - lean_ctor_release(x_89, 0); - lean_ctor_release(x_89, 1); - x_92 = x_89; +lean_dec(x_6); +lean_dec(x_5); +x_194 = lean_ctor_get(x_147, 0); +lean_inc(x_194); +x_195 = lean_ctor_get(x_147, 1); +lean_inc(x_195); +if (lean_is_exclusive(x_147)) { + lean_ctor_release(x_147, 0); + lean_ctor_release(x_147, 1); + x_196 = x_147; } else { - lean_dec_ref(x_89); - x_92 = lean_box(0); + lean_dec_ref(x_147); + x_196 = lean_box(0); } -if (lean_is_scalar(x_92)) { - x_93 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_196)) { + x_197 = lean_alloc_ctor(1, 2, 0); } else { - x_93 = x_92; + x_197 = x_196; +} +lean_ctor_set(x_197, 0, x_194); +lean_ctor_set(x_197, 1, x_195); +return x_197; } -lean_ctor_set(x_93, 0, x_90); -lean_ctor_set(x_93, 1, x_91); -return x_93; } } +block_19: +{ +size_t x_16; size_t x_17; +x_16 = 1; +x_17 = lean_usize_add(x_2, x_16); +x_2 = x_17; +x_4 = x_14; +x_11 = x_15; +goto _start; +} } else { -lean_object* x_94; +lean_object* x_198; 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_94 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_94, 0, x_4); -lean_ctor_set(x_94, 1, x_11); -return x_94; +x_198 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_198, 0, x_4); +lean_ctor_set(x_198, 1, x_11); +return x_198; } } } @@ -27733,7 +26513,6 @@ lean_dec(x_2); x_13 = lean_unbox_usize(x_3); lean_dec(x_3); x_14 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___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_6); lean_dec(x_1); return x_14; } @@ -27766,7 +26545,7 @@ static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_s lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__1; x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_setSourceInstImplicit___closed__1; -x_3 = lean_unsigned_to_nat(768u); +x_3 = lean_unsigned_to_nat(842u); x_4 = lean_unsigned_to_nat(9u); x_5 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -28042,7 +26821,7 @@ x_19 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_ x_20 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_20, 0, x_19); lean_ctor_set(x_20, 1, x_18); -x_21 = l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__4; +x_21 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3; x_22 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_22, 0, x_20); lean_ctor_set(x_22, 1, x_21); @@ -28154,7 +26933,7 @@ static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Stru lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__1; x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent_copyFields___spec__2___closed__1; -x_3 = lean_unsigned_to_nat(792u); +x_3 = lean_unsigned_to_nat(865u); x_4 = lean_unsigned_to_nat(79u); x_5 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -28202,7 +26981,7 @@ else { lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_26; x_16 = lean_array_uget(x_5, x_7); -x_26 = l_Array_contains___at_Lean_findField_x3f___spec__1(x_2, x_16); +x_26 = l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(x_2, x_16); if (x_26 == 0) { lean_object* x_27; @@ -28455,7 +27234,7 @@ static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_m lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__1; x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent_copyFields___spec__2___closed__1; -x_3 = lean_unsigned_to_nat(783u); +x_3 = lean_unsigned_to_nat(856u); x_4 = lean_unsigned_to_nat(70u); x_5 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -28487,7 +27266,7 @@ 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___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; +x_19 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__4; lean_inc(x_18); x_20 = lean_mk_array(x_18, x_19); x_21 = lean_unsigned_to_nat(1u); @@ -28696,8 +27475,8 @@ x_43 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_43, 0, x_42); lean_ctor_set(x_43, 1, x_8); lean_ctor_set(x_43, 2, x_21); -x_44 = lean_ctor_get(x_9, 1); -x_45 = lean_ctor_get_uint8(x_44, sizeof(void*)*2 + 3); +x_44 = lean_ctor_get(x_9, 2); +x_45 = lean_ctor_get_uint8(x_44, sizeof(void*)*3 + 3); lean_inc(x_42); lean_ctor_set_tag(x_33, 1); lean_ctor_set(x_33, 1, x_10); @@ -28908,8 +27687,8 @@ x_90 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_90, 0, x_89); lean_ctor_set(x_90, 1, x_8); lean_ctor_set(x_90, 2, x_21); -x_91 = lean_ctor_get(x_9, 1); -x_92 = lean_ctor_get_uint8(x_91, sizeof(void*)*2 + 3); +x_91 = lean_ctor_get(x_9, 2); +x_92 = lean_ctor_get_uint8(x_91, sizeof(void*)*3 + 3); lean_inc(x_89); x_93 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_93, 0, x_89); @@ -29331,29 +28110,8 @@ return x_45; } } } -} -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("_private.Lean.Elab.Structure.0.Lean.Elab.Command.mkCoercionToCopiedParent", 73, 73); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__1; -x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___closed__1; -x_3 = lean_unsigned_to_nat(775u); -x_4 = lean_unsigned_to_nat(65u); -x_5 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___closed__3; -x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); -return x_6; -} -} -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___closed__3() { +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___closed__1() { _start: { lean_object* x_1; @@ -29361,144 +28119,120 @@ x_1 = lean_mk_string_unchecked("self", 4, 4); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___closed__4() { +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___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_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___closed__3; +x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_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_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_10; lean_object* x_11; 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; -x_10 = lean_st_ref_get(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_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; uint8_t x_23; +x_11 = lean_st_ref_get(x_9, x_10); +x_12 = lean_ctor_get(x_11, 0); lean_inc(x_12); -lean_dec(x_10); -x_13 = lean_ctor_get(x_11, 0); +x_13 = lean_ctor_get(x_11, 1); lean_inc(x_13); lean_dec(x_11); -x_14 = lean_ctor_get(x_3, 4); -lean_inc(x_14); -x_15 = 1; +x_14 = lean_ctor_get(x_12, 0); lean_inc(x_14); -x_16 = l_Lean_getStructureFieldsFlattened(x_13, x_14, x_15); -x_17 = lean_box(0); +lean_dec(x_12); +x_15 = lean_ctor_get(x_3, 4); +lean_inc(x_15); +x_16 = 1; +lean_inc(x_15); +x_17 = l_Lean_getStructureFieldsFlattened(x_14, x_15, x_16); +x_18 = lean_box(0); lean_inc(x_1); -x_18 = l_List_mapTR_loop___at_Lean_mkConstWithLevelParams___spec__1(x_1, x_17); -lean_inc(x_14); -x_19 = l_Lean_Expr_const___override(x_14, x_18); -x_20 = l_Lean_mkAppN(x_19, x_2); -x_21 = l_Lean_Expr_getAppFn(x_4); -if (lean_obj_tag(x_21) == 4) -{ -lean_object* x_22; uint8_t x_23; uint8_t x_24; -x_22 = lean_ctor_get(x_21, 0); -lean_inc(x_22); -lean_dec(x_21); -x_23 = lean_ctor_get_uint8(x_3, sizeof(void*)*11); -if (x_23 == 0) +x_19 = l_List_mapTR_loop___at_Lean_mkConstWithLevelParams___spec__1(x_1, x_18); +lean_inc(x_15); +x_20 = l_Lean_Expr_const___override(x_15, x_19); +x_21 = l_Lean_mkAppN(x_20, x_2); +x_22 = lean_ctor_get_uint8(x_3, sizeof(void*)*12); +if (x_22 == 0) { -uint8_t x_44; -lean_dec(x_22); -x_44 = 0; -x_24 = x_44; -goto block_43; +uint8_t x_43; +lean_dec(x_4); +x_43 = 0; +x_23 = x_43; +goto block_42; } else { -uint8_t x_45; -lean_inc(x_13); -x_45 = lean_is_class(x_13, x_22); -x_24 = x_45; -goto block_43; +uint8_t x_44; +lean_inc(x_14); +x_44 = lean_is_class(x_14, x_4); +x_23 = x_44; +goto block_42; } -block_43: +block_42: { -uint8_t x_25; -if (x_24 == 0) +uint8_t x_24; +if (x_23 == 0) { -uint8_t x_42; -x_42 = 0; -x_25 = x_42; -goto block_41; +uint8_t x_41; +x_41 = 0; +x_24 = x_41; +goto block_40; } else { -x_25 = x_15; -goto block_41; +x_24 = x_16; +goto block_40; } -block_41: +block_40: { -if (x_25 == 0) +if (x_24 == 0) { -uint8_t 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_26 = 0; -x_27 = lean_box(x_26); -x_28 = lean_box(x_25); -x_29 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___lambda__3___boxed), 16, 10); -lean_closure_set(x_29, 0, x_17); -lean_closure_set(x_29, 1, x_4); -lean_closure_set(x_29, 2, x_2); -lean_closure_set(x_29, 3, x_13); -lean_closure_set(x_29, 4, x_16); -lean_closure_set(x_29, 5, x_14); -lean_closure_set(x_29, 6, x_1); -lean_closure_set(x_29, 7, x_3); -lean_closure_set(x_29, 8, x_27); -lean_closure_set(x_29, 9, x_28); -x_30 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___closed__4; -x_31 = 0; -x_32 = l_Lean_Meta_withLocalDecl___at_Lean_Meta_GeneralizeTelescope_generalizeTelescopeAux___spec__1___rarg(x_30, x_26, x_20, x_29, x_31, x_5, x_6, x_7, x_8, x_12); -return x_32; +uint8_t x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; lean_object* x_31; +x_25 = 0; +x_26 = lean_box(x_25); +x_27 = lean_box(x_24); +x_28 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___lambda__3___boxed), 16, 10); +lean_closure_set(x_28, 0, x_18); +lean_closure_set(x_28, 1, x_5); +lean_closure_set(x_28, 2, x_2); +lean_closure_set(x_28, 3, x_14); +lean_closure_set(x_28, 4, x_17); +lean_closure_set(x_28, 5, x_15); +lean_closure_set(x_28, 6, x_1); +lean_closure_set(x_28, 7, x_3); +lean_closure_set(x_28, 8, x_26); +lean_closure_set(x_28, 9, x_27); +x_29 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___closed__2; +x_30 = 0; +x_31 = l_Lean_Meta_withLocalDecl___at_Lean_Meta_GeneralizeTelescope_generalizeTelescopeAux___spec__1___rarg(x_29, x_25, x_21, x_28, x_30, x_6, x_7, x_8, x_9, x_13); +return x_31; } else { -uint8_t x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; uint8_t x_38; uint8_t x_39; lean_object* x_40; -x_33 = 3; -x_34 = lean_box(x_33); -x_35 = lean_box(x_25); -x_36 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___lambda__3___boxed), 16, 10); -lean_closure_set(x_36, 0, x_17); -lean_closure_set(x_36, 1, x_4); -lean_closure_set(x_36, 2, x_2); -lean_closure_set(x_36, 3, x_13); -lean_closure_set(x_36, 4, x_16); -lean_closure_set(x_36, 5, x_14); -lean_closure_set(x_36, 6, x_1); -lean_closure_set(x_36, 7, x_3); -lean_closure_set(x_36, 8, x_34); -lean_closure_set(x_36, 9, x_35); -x_37 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___closed__4; +uint8_t x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; uint8_t x_38; lean_object* x_39; +x_32 = 3; +x_33 = lean_box(x_32); +x_34 = lean_box(x_24); +x_35 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___lambda__3___boxed), 16, 10); +lean_closure_set(x_35, 0, x_18); +lean_closure_set(x_35, 1, x_5); +lean_closure_set(x_35, 2, x_2); +lean_closure_set(x_35, 3, x_14); +lean_closure_set(x_35, 4, x_17); +lean_closure_set(x_35, 5, x_15); +lean_closure_set(x_35, 6, x_1); +lean_closure_set(x_35, 7, x_3); +lean_closure_set(x_35, 8, x_33); +lean_closure_set(x_35, 9, x_34); +x_36 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___closed__2; +x_37 = 0; x_38 = 0; -x_39 = 0; -x_40 = l_Lean_Meta_withLocalDecl___at_Lean_Meta_GeneralizeTelescope_generalizeTelescopeAux___spec__1___rarg(x_37, x_38, x_20, x_36, x_39, x_5, x_6, x_7, x_8, x_12); -return x_40; -} -} +x_39 = l_Lean_Meta_withLocalDecl___at_Lean_Meta_GeneralizeTelescope_generalizeTelescopeAux___spec__1___rarg(x_36, x_37, x_21, x_35, x_38, x_6, x_7, x_8, x_9, x_13); +return x_39; } } -else -{ -lean_object* x_46; lean_object* x_47; -lean_dec(x_21); -lean_dec(x_20); -lean_dec(x_16); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_46 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___closed__2; -x_47 = l_panic___at_Lean_mkNoConfusionEnum_mkToCtorIdx___spec__1(x_46, x_5, x_6, x_7, x_8, x_12); -return x_47; } } } @@ -29556,598 +28290,897 @@ lean_dec(x_5); return x_19; } } -LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__1(lean_object* x_1, lean_object* x_2) { _start: { -if (lean_obj_tag(x_1) == 0) +lean_object* x_3; uint8_t x_4; +x_3 = lean_ctor_get(x_1, 3); +x_4 = lean_name_eq(x_3, x_2); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___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_3; -x_3 = l_List_reverse___rarg(x_2); -return x_3; +lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_15 = lean_ctor_get(x_10, 1); +x_16 = l_Lean_Meta_getLocalInstances(x_10, x_11, x_12, x_13, x_14); +x_17 = !lean_is_exclusive(x_16); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; +x_18 = lean_ctor_get(x_16, 0); +lean_inc(x_15); +x_19 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_19, 0, x_1); +lean_ctor_set(x_19, 1, x_15); +lean_ctor_set(x_19, 2, x_18); +lean_ctor_set(x_19, 3, x_2); +lean_ctor_set(x_19, 4, x_3); +lean_ctor_set(x_19, 5, x_4); +lean_ctor_set(x_19, 6, x_5); +lean_ctor_set(x_19, 7, x_6); +lean_ctor_set(x_16, 0, x_19); +return x_16; } else { -uint8_t x_4; -x_4 = !lean_is_exclusive(x_1); -if (x_4 == 0) +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +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); +lean_inc(x_15); +x_22 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_22, 0, x_1); +lean_ctor_set(x_22, 1, x_15); +lean_ctor_set(x_22, 2, x_20); +lean_ctor_set(x_22, 3, x_2); +lean_ctor_set(x_22, 4, x_3); +lean_ctor_set(x_22, 5, x_4); +lean_ctor_set(x_22, 6, x_5); +lean_ctor_set(x_22, 7, x_6); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_21); +return x_23; +} +} +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__1() { +_start: { -lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_5 = lean_ctor_get(x_1, 0); -x_6 = lean_ctor_get(x_1, 1); -x_7 = lean_ctor_get(x_5, 1); -lean_inc(x_7); -lean_dec(x_5); -lean_ctor_set(x_1, 1, x_2); -lean_ctor_set(x_1, 0, x_7); +lean_object* x_1; +x_1 = lean_mk_string_unchecked("header params: ", 15, 15); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__2() { +_start: { -lean_object* _tmp_0 = x_6; -lean_object* _tmp_1 = x_1; -x_1 = _tmp_0; -x_2 = _tmp_1; +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } -goto _start; +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(", type: ", 8, 8); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(", levelNames: ", 14, 14); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__5; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; uint8_t x_14; +x_13 = l_Lean_Elab_Term_getLevelNames___rarg(x_7, x_8, x_9, x_10, x_11, x_12); +x_14 = !lean_is_exclusive(x_13); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; +x_15 = lean_ctor_get(x_13, 0); +x_16 = lean_ctor_get(x_13, 1); +x_17 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__1; +x_18 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_17, x_6, x_7, x_8, x_9, x_10, x_11, x_16); +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +x_20 = lean_unbox(x_19); +lean_dec(x_19); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; +lean_free_object(x_13); +x_21 = lean_ctor_get(x_18, 1); +lean_inc(x_21); +lean_dec(x_18); +x_22 = lean_box(0); +x_23 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__2(x_1, x_15, x_4, x_5, x_2, x_3, x_22, x_6, x_7, x_8, x_9, x_10, x_11, x_21); +return x_23; } else { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_9 = lean_ctor_get(x_1, 0); -x_10 = lean_ctor_get(x_1, 1); -lean_inc(x_10); -lean_inc(x_9); -lean_dec(x_1); -x_11 = lean_ctor_get(x_9, 1); -lean_inc(x_11); -lean_dec(x_9); -x_12 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_12, 0, x_11); -lean_ctor_set(x_12, 1, x_2); -x_1 = x_10; -x_2 = x_12; -goto _start; +uint8_t x_24; +x_24 = !lean_is_exclusive(x_18); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; 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_25 = lean_ctor_get(x_18, 1); +x_26 = lean_ctor_get(x_18, 0); +lean_dec(x_26); +lean_inc(x_4); +x_27 = lean_array_to_list(x_4); +x_28 = lean_box(0); +x_29 = l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(x_27, x_28); +x_30 = l_Lean_MessageData_ofList(x_29); +x_31 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__2; +lean_ctor_set_tag(x_18, 7); +lean_ctor_set(x_18, 1, x_30); +lean_ctor_set(x_18, 0, x_31); +x_32 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__4; +lean_ctor_set_tag(x_13, 7); +lean_ctor_set(x_13, 1, x_32); +lean_ctor_set(x_13, 0, x_18); +lean_inc(x_5); +x_33 = l_Lean_MessageData_ofExpr(x_5); +x_34 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_34, 0, x_13); +lean_ctor_set(x_34, 1, x_33); +x_35 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__6; +x_36 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_36, 0, x_34); +lean_ctor_set(x_36, 1, x_35); +lean_inc(x_15); +x_37 = l_List_mapTR_loop___at_Lean_compileDecl___spec__1(x_15, x_28); +x_38 = l_Lean_MessageData_ofList(x_37); +x_39 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_39, 0, x_36); +lean_ctor_set(x_39, 1, x_38); +x_40 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3; +x_41 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_41, 0, x_39); +lean_ctor_set(x_41, 1, x_40); +x_42 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_17, x_41, x_6, x_7, x_8, x_9, x_10, x_11, x_25); +x_43 = lean_ctor_get(x_42, 0); +lean_inc(x_43); +x_44 = lean_ctor_get(x_42, 1); +lean_inc(x_44); +lean_dec(x_42); +x_45 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__2(x_1, x_15, x_4, x_5, x_2, x_3, x_43, x_6, x_7, x_8, x_9, x_10, x_11, x_44); +lean_dec(x_43); +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; 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_46 = lean_ctor_get(x_18, 1); +lean_inc(x_46); +lean_dec(x_18); +lean_inc(x_4); +x_47 = lean_array_to_list(x_4); +x_48 = lean_box(0); +x_49 = l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(x_47, x_48); +x_50 = l_Lean_MessageData_ofList(x_49); +x_51 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__2; +x_52 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_52, 0, x_51); +lean_ctor_set(x_52, 1, x_50); +x_53 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__4; +lean_ctor_set_tag(x_13, 7); +lean_ctor_set(x_13, 1, x_53); +lean_ctor_set(x_13, 0, x_52); +lean_inc(x_5); +x_54 = l_Lean_MessageData_ofExpr(x_5); +x_55 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_55, 0, x_13); +lean_ctor_set(x_55, 1, x_54); +x_56 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__6; +x_57 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_57, 0, x_55); +lean_ctor_set(x_57, 1, x_56); +lean_inc(x_15); +x_58 = l_List_mapTR_loop___at_Lean_compileDecl___spec__1(x_15, x_48); +x_59 = l_Lean_MessageData_ofList(x_58); +x_60 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_60, 0, x_57); +lean_ctor_set(x_60, 1, x_59); +x_61 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3; +x_62 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_62, 0, x_60); +lean_ctor_set(x_62, 1, x_61); +x_63 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_17, x_62, x_6, x_7, x_8, x_9, x_10, x_11, x_46); +x_64 = lean_ctor_get(x_63, 0); +lean_inc(x_64); +x_65 = lean_ctor_get(x_63, 1); +lean_inc(x_65); +lean_dec(x_63); +x_66 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__2(x_1, x_15, x_4, x_5, x_2, x_3, x_64, x_6, x_7, x_8, x_9, x_10, x_11, x_65); +lean_dec(x_64); +return x_66; +} +} +} +else +{ +lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; uint8_t x_72; +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 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__1; +x_70 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_69, x_6, x_7, x_8, x_9, x_10, x_11, x_68); +x_71 = lean_ctor_get(x_70, 0); +lean_inc(x_71); +x_72 = lean_unbox(x_71); +lean_dec(x_71); +if (x_72 == 0) +{ +lean_object* x_73; lean_object* x_74; lean_object* x_75; +x_73 = lean_ctor_get(x_70, 1); +lean_inc(x_73); +lean_dec(x_70); +x_74 = lean_box(0); +x_75 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__2(x_1, x_67, x_4, x_5, x_2, x_3, x_74, x_6, x_7, x_8, x_9, x_10, x_11, x_73); +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_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; +x_76 = lean_ctor_get(x_70, 1); +lean_inc(x_76); +if (lean_is_exclusive(x_70)) { + lean_ctor_release(x_70, 0); + lean_ctor_release(x_70, 1); + x_77 = x_70; +} else { + lean_dec_ref(x_70); + x_77 = lean_box(0); +} +lean_inc(x_4); +x_78 = lean_array_to_list(x_4); +x_79 = lean_box(0); +x_80 = l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(x_78, x_79); +x_81 = l_Lean_MessageData_ofList(x_80); +x_82 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__2; +if (lean_is_scalar(x_77)) { + x_83 = lean_alloc_ctor(7, 2, 0); +} else { + x_83 = x_77; + lean_ctor_set_tag(x_83, 7); +} +lean_ctor_set(x_83, 0, x_82); +lean_ctor_set(x_83, 1, x_81); +x_84 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__4; +x_85 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_85, 0, x_83); +lean_ctor_set(x_85, 1, x_84); +lean_inc(x_5); +x_86 = l_Lean_MessageData_ofExpr(x_5); +x_87 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_87, 0, x_85); +lean_ctor_set(x_87, 1, x_86); +x_88 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__6; +x_89 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_89, 0, x_87); +lean_ctor_set(x_89, 1, x_88); +lean_inc(x_67); +x_90 = l_List_mapTR_loop___at_Lean_compileDecl___spec__1(x_67, x_79); +x_91 = l_Lean_MessageData_ofList(x_90); +x_92 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_92, 0, x_89); +lean_ctor_set(x_92, 1, x_91); +x_93 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3; +x_94 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_94, 0, x_92); +lean_ctor_set(x_94, 1, x_93); +x_95 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_69, x_94, x_6, x_7, x_8, x_9, x_10, x_11, x_76); +x_96 = lean_ctor_get(x_95, 0); +lean_inc(x_96); +x_97 = lean_ctor_get(x_95, 1); +lean_inc(x_97); +lean_dec(x_95); +x_98 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__2(x_1, x_67, x_4, x_5, x_2, x_3, x_96, x_6, x_7, x_8, x_9, x_10, x_11, x_97); +lean_dec(x_96); +return x_98; } } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__2(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_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_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -uint8_t x_12; -x_12 = lean_usize_dec_lt(x_3, x_2); -if (x_12 == 0) +lean_object* x_14; +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +x_14 = lean_whnf(x_1, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_14) == 0) { -lean_object* 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; +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_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_15, x_7, x_8, x_9, x_10, x_11, x_12, x_16); +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); +lean_dec(x_17); +x_20 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___boxed), 12, 3); +lean_closure_set(x_20, 0, x_2); +lean_closure_set(x_20, 1, x_3); +lean_closure_set(x_20, 2, x_4); +x_21 = l_Lean_Elab_Term_addAutoBoundImplicits_x27___rarg(x_5, x_18, x_20, x_7, x_8, x_9, x_10, x_11, x_12, x_19); +return x_21; +} +else +{ +uint8_t x_22; +lean_dec(x_12); +lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -x_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; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_22 = !lean_is_exclusive(x_14); +if (x_22 == 0) +{ +return x_14; } else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; -lean_dec(x_4); -x_14 = lean_array_uget(x_1, x_3); -x_15 = lean_st_ref_get(x_10, x_11); -x_16 = lean_ctor_get(x_15, 0); -lean_inc(x_16); -x_17 = lean_ctor_get(x_15, 1); -lean_inc(x_17); -lean_dec(x_15); -x_18 = lean_ctor_get(x_16, 0); -lean_inc(x_18); -lean_dec(x_16); -x_19 = lean_ctor_get(x_14, 2); -lean_inc(x_19); -x_20 = l_Lean_Environment_contains(x_18, x_19); -if (x_20 == 0) -{ -size_t x_21; size_t x_22; lean_object* x_23; -lean_dec(x_19); +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_14, 0); +x_24 = lean_ctor_get(x_14, 1); +lean_inc(x_24); +lean_inc(x_23); lean_dec(x_14); -x_21 = 1; -x_22 = lean_usize_add(x_3, x_21); -x_23 = lean_box(0); -x_3 = x_22; -x_4 = x_23; -x_11 = x_17; -goto _start; +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 +} +} +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__5___closed__1() { +_start: { -lean_object* x_25; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("invalid structure type, expecting 'Type _' or 'Prop'", 52, 52); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__5___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__5___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; lean_object* x_13; +x_12 = lean_ctor_get(x_1, 7); +lean_inc(x_12); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); lean_inc(x_5); -x_25 = l_Lean_mkConstWithLevelParams___at_Lean_Elab_Term_expandDeclId___spec__7(x_19, x_5, x_6, x_7, x_8, x_9, x_10, x_17); -if (lean_obj_tag(x_25) == 0) +lean_inc(x_12); +x_13 = l_Lean_Elab_Term_elabType(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_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_26 = lean_ctor_get(x_25, 0); -lean_inc(x_26); -x_27 = lean_ctor_get(x_25, 1); -lean_inc(x_27); -lean_dec(x_25); -x_28 = lean_ctor_get(x_14, 0); -lean_inc(x_28); -lean_dec(x_14); -x_29 = lean_box(0); -x_30 = lean_box(0); -x_31 = 1; +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_13, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_13, 1); +lean_inc(x_15); +lean_dec(x_13); +x_16 = 1; +x_17 = 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_32 = l_Lean_Elab_Term_addTermInfo_x27(x_28, x_26, x_29, x_29, x_30, x_31, x_5, x_6, x_7, x_8, x_9, x_10, x_27); -if (lean_obj_tag(x_32) == 0) +x_18 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_16, x_17, x_5, x_6, x_7, x_8, x_9, x_10, x_15); +if (lean_obj_tag(x_18) == 0) { -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_3, x_34); -x_36 = lean_box(0); -x_3 = x_35; -x_4 = x_36; -x_11 = x_33; -goto _start; -} -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; +x_19 = lean_ctor_get(x_18, 1); +lean_inc(x_19); +lean_dec(x_18); +x_20 = l_Lean_Meta_mkFreshLevelMVar(x_7, x_8, x_9, x_10, x_19); +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +x_23 = l_Lean_Expr_sort___override(x_21); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_14); +x_24 = l_Lean_Meta_isExprDefEq(x_14, x_23, x_7, x_8, x_9, x_10, x_22); +if (lean_obj_tag(x_24) == 0) { -uint8_t x_38; +lean_object* x_25; uint8_t x_26; +x_25 = lean_ctor_get(x_24, 0); +lean_inc(x_25); +x_26 = lean_unbox(x_25); +lean_dec(x_25); +if (x_26 == 0) +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; +lean_dec(x_14); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_27 = lean_ctor_get(x_24, 1); +lean_inc(x_27); +lean_dec(x_24); +x_28 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__5___closed__2; +x_29 = l_Lean_throwErrorAt___at___private_Lean_Elab_Binders_0__Lean_Elab_Term_elabBinderViews_loop___spec__1(x_12, x_28, 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); -x_38 = !lean_is_exclusive(x_32); -if (x_38 == 0) +lean_dec(x_12); +x_30 = !lean_is_exclusive(x_29); +if (x_30 == 0) { -return x_32; +return x_29; } else { -lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_39 = lean_ctor_get(x_32, 0); -x_40 = lean_ctor_get(x_32, 1); -lean_inc(x_40); -lean_inc(x_39); -lean_dec(x_32); -x_41 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_41, 0, x_39); -lean_ctor_set(x_41, 1, x_40); -return x_41; +lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_31 = lean_ctor_get(x_29, 0); +x_32 = lean_ctor_get(x_29, 1); +lean_inc(x_32); +lean_inc(x_31); +lean_dec(x_29); +x_33 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_33, 0, x_31); +lean_ctor_set(x_33, 1, x_32); +return x_33; } } +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; +lean_dec(x_12); +x_34 = lean_ctor_get(x_24, 1); +lean_inc(x_34); +lean_dec(x_24); +x_35 = lean_box(0); +x_36 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__4(x_14, x_1, x_4, x_3, x_2, x_35, x_5, x_6, x_7, x_8, x_9, x_10, x_34); +return x_36; +} } else { -uint8_t x_42; +uint8_t x_37; lean_dec(x_14); +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_42 = !lean_is_exclusive(x_25); -if (x_42 == 0) +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_37 = !lean_is_exclusive(x_24); +if (x_37 == 0) { -return x_25; +return x_24; } else { -lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_43 = lean_ctor_get(x_25, 0); -x_44 = lean_ctor_get(x_25, 1); -lean_inc(x_44); -lean_inc(x_43); -lean_dec(x_25); -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_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_24, 0); +x_39 = lean_ctor_get(x_24, 1); +lean_inc(x_39); +lean_inc(x_38); +lean_dec(x_24); +x_40 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +return x_40; } } } -LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___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: -{ -if (lean_obj_tag(x_1) == 0) +else { -lean_object* x_9; lean_object* x_10; +uint8_t x_41; +lean_dec(x_14); +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); -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; +lean_dec(x_3); +lean_dec(x_1); +x_41 = !lean_is_exclusive(x_18); +if (x_41 == 0) +{ +return x_18; } else { -lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; lean_object* 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); -lean_dec(x_1); -x_13 = 0; -x_14 = lean_unsigned_to_nat(1000u); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -x_15 = l_Lean_Meta_addInstance(x_11, x_13, x_14, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_15) == 0) -{ -lean_object* x_16; -x_16 = lean_ctor_get(x_15, 1); -lean_inc(x_16); -lean_dec(x_15); -x_1 = x_12; -x_8 = x_16; -goto _start; +lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_42 = lean_ctor_get(x_18, 0); +x_43 = lean_ctor_get(x_18, 1); +lean_inc(x_43); +lean_inc(x_42); +lean_dec(x_18); +x_44 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_44, 0, x_42); +lean_ctor_set(x_44, 1, x_43); +return x_44; +} +} } else { -uint8_t x_18; +uint8_t x_45; 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); -x_18 = !lean_is_exclusive(x_15); -if (x_18 == 0) +lean_dec(x_3); +lean_dec(x_1); +x_45 = !lean_is_exclusive(x_13); +if (x_45 == 0) { -return x_15; +return x_13; } else { -lean_object* x_19; lean_object* x_20; lean_object* x_21; -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(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_46; lean_object* x_47; lean_object* x_48; +x_46 = lean_ctor_get(x_13, 0); +x_47 = lean_ctor_get(x_13, 1); +lean_inc(x_47); +lean_inc(x_46); +lean_dec(x_13); +x_48 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_48, 0, x_46); +lean_ctor_set(x_48, 1, x_47); +return x_48; } } -static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__4___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Init.Data.Option.BasicAux", 25, 25); -return x_1; } } -static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__4___closed__2() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Option.get!", 11, 11); -return x_1; +lean_object* x_10; lean_object* x_11; +lean_inc(x_1); +x_10 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__5___boxed), 11, 2); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, x_2); +x_11 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents___rarg(x_1, x_10, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_11; } } -static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__4___closed__3() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader(lean_object* x_1, lean_object* x_2, lean_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_unchecked("value is none", 13, 13); -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_inc(x_1); +x_9 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__1___boxed), 2, 1); +lean_closure_set(x_9, 0, x_1); +x_10 = lean_ctor_get(x_1, 6); +lean_inc(x_10); +x_11 = l_Lean_Syntax_getArgs(x_10); +lean_dec(x_10); +x_12 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__6), 9, 1); +lean_closure_set(x_12, 0, x_1); +x_13 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabBinders___rarg), 9, 2); +lean_closure_set(x_13, 0, x_11); +lean_closure_set(x_13, 1, x_12); +x_14 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withAutoBoundImplicit___rarg), 8, 1); +lean_closure_set(x_14, 0, x_13); +x_15 = l_Lean_Elab_Term_withAutoBoundImplicitForbiddenPred___rarg(x_9, x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +return x_15; } } -static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__4___closed__4() { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__1___boxed(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; lean_object* x_5; lean_object* x_6; -x_1 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__4___closed__1; -x_2 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__4___closed__2; -x_3 = lean_unsigned_to_nat(16u); -x_4 = lean_unsigned_to_nat(14u); -x_5 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__4___closed__3; -x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); -return x_6; +uint8_t x_3; lean_object* x_4; +x_3 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__1(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +x_4 = lean_box(x_3); +return x_4; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___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) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { -uint8_t x_11; -x_11 = lean_usize_dec_lt(x_2, x_1); -if (x_11 == 0) -{ -lean_object* x_12; +lean_object* x_15; +x_15 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); -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; lean_object* x_17; -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, 2); -lean_inc(x_16); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -x_17 = lean_infer_type(x_16, 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; lean_object* x_22; -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_17, 1); -lean_inc(x_19); -lean_dec(x_17); -x_20 = lean_ctor_get(x_13, 1); -lean_inc(x_20); -x_21 = l_Lean_mkDefaultFnOfProjFn(x_20); -x_22 = lean_ctor_get(x_13, 3); -lean_inc(x_22); -lean_dec(x_13); -if (lean_obj_tag(x_22) == 0) -{ -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; size_t x_27; size_t x_28; lean_object* x_29; -x_23 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__4___closed__4; -x_24 = l_panic___at_Lean_Expr_appFn_x21___spec__1(x_23); -x_25 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_25, 0, x_18); -lean_ctor_set(x_25, 1, x_24); -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_21); -lean_ctor_set(x_26, 1, x_25); -x_27 = 1; -x_28 = lean_usize_add(x_2, x_27); -x_29 = lean_array_uset(x_15, x_2, x_26); -x_2 = x_28; -x_3 = x_29; -x_10 = x_19; -goto _start; -} -else -{ -lean_object* x_31; lean_object* x_32; lean_object* x_33; size_t x_34; size_t x_35; lean_object* x_36; -x_31 = lean_ctor_get(x_22, 0); -lean_inc(x_31); -lean_dec(x_22); -x_32 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_32, 0, x_18); -lean_ctor_set(x_32, 1, x_31); -x_33 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_33, 0, x_21); -lean_ctor_set(x_33, 1, x_32); -x_34 = 1; -x_35 = lean_usize_add(x_2, x_34); -x_36 = lean_array_uset(x_15, x_2, x_33); -x_2 = x_35; -x_3 = x_36; -x_10 = x_19; -goto _start; +return x_15; } } -else +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: { -uint8_t x_38; -lean_dec(x_15); -lean_dec(x_13); +lean_object* x_13; +x_13 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_11); +lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -x_38 = !lean_is_exclusive(x_17); -if (x_38 == 0) -{ -return x_17; -} -else -{ -lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_39 = lean_ctor_get(x_17, 0); -x_40 = lean_ctor_get(x_17, 1); -lean_inc(x_40); -lean_inc(x_39); -lean_dec(x_17); -x_41 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_41, 0, x_39); -lean_ctor_set(x_41, 1, x_40); -return x_41; -} -} -} +return x_13; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__5(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -uint8_t x_5; -x_5 = lean_usize_dec_eq(x_2, x_3); -if (x_5 == 0) -{ -lean_object* x_6; uint8_t x_7; size_t x_8; size_t x_9; -x_6 = lean_array_uget(x_1, x_2); -x_7 = l_Lean_Elab_Command_StructFieldInfo_isFromParent(x_6); -x_8 = 1; -x_9 = lean_usize_add(x_2, x_8); -if (x_7 == 0) -{ -lean_object* x_10; lean_object* x_11; uint8_t x_12; lean_object* x_13; -x_10 = lean_ctor_get(x_6, 2); -lean_inc(x_10); -lean_dec(x_6); -x_11 = l_Lean_Expr_fvarId_x21(x_10); -lean_dec(x_10); -x_12 = 0; -x_13 = l_Lean_LocalContext_setBinderInfo(x_4, x_11, x_12); -x_2 = x_9; -x_4 = x_13; -goto _start; -} -else -{ +lean_object* x_14; +x_14 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); lean_dec(x_6); -x_2 = x_9; -goto _start; -} -} -else -{ -return x_4; -} +lean_dec(x_5); +return x_14; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__6(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -uint8_t x_5; -x_5 = lean_usize_dec_eq(x_2, x_3); -if (x_5 == 0) -{ -lean_object* x_6; uint8_t x_7; size_t x_8; size_t x_9; -x_6 = lean_array_uget(x_1, x_2); -x_7 = l_Lean_Expr_isFVar(x_6); -x_8 = 1; -x_9 = lean_usize_add(x_2, x_8); -if (x_7 == 0) -{ -lean_dec(x_6); -x_2 = x_9; -goto _start; +lean_object* x_12; +x_12 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_2); +return x_12; } -else +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkTypeFor___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_11; uint8_t x_12; lean_object* x_13; -x_11 = l_Lean_Expr_fvarId_x21(x_6); -lean_dec(x_6); +uint8_t x_10; uint8_t x_11; uint8_t x_12; lean_object* x_13; +x_10 = 0; +x_11 = 1; x_12 = 1; -x_13 = l_Lean_LocalContext_setBinderInfo(x_4, x_11, x_12); -x_2 = x_9; -x_4 = x_13; -goto _start; +x_13 = l_Lean_Meta_mkForallFVars(x_1, x_2, x_10, x_11, x_12, x_5, x_6, x_7, x_8, x_9); +return x_13; } } -else +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkTypeFor(lean_object* x_1, lean_object* x_2, lean_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_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 = lean_ctor_get(x_1, 2); +lean_inc(x_10); +x_11 = lean_ctor_get(x_1, 4); +lean_inc(x_11); +x_12 = lean_ctor_get(x_1, 5); +lean_inc(x_12); +lean_dec(x_1); +x_13 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkTypeFor___lambda__1___boxed), 9, 2); +lean_closure_set(x_13, 0, x_11); +lean_closure_set(x_13, 1, x_12); +x_14 = l_Lean_Meta_withLCtx___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__3___rarg(x_9, x_10, x_13, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +return x_14; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__7(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkTypeFor___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, 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_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 = lean_ctor_get(x_6, 3); -lean_inc(x_7); -x_8 = 1; -x_9 = lean_usize_add(x_2, x_8); -if (lean_obj_tag(x_7) == 0) -{ +lean_object* x_10; +x_10 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkTypeFor___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); -x_2 = x_9; -goto _start; +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_10; } -else -{ -lean_object* x_11; -lean_dec(x_7); -x_11 = lean_array_push(x_4, x_6); -x_2 = x_9; -x_4 = x_11; -goto _start; } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withStructureLocalDecl___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: +{ +uint8_t x_13; +x_13 = !lean_is_exclusive(x_10); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_10, 5); +x_15 = l_Lean_replaceRef(x_1, x_14); +lean_dec(x_14); +lean_ctor_set(x_10, 5, x_15); +x_16 = l_Lean_Elab_Term_withAuxDecl___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +return x_16; } else { -return x_4; +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; uint8_t x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_17 = lean_ctor_get(x_10, 0); +x_18 = lean_ctor_get(x_10, 1); +x_19 = lean_ctor_get(x_10, 2); +x_20 = lean_ctor_get(x_10, 3); +x_21 = lean_ctor_get(x_10, 4); +x_22 = lean_ctor_get(x_10, 5); +x_23 = lean_ctor_get(x_10, 6); +x_24 = lean_ctor_get(x_10, 7); +x_25 = lean_ctor_get(x_10, 8); +x_26 = lean_ctor_get(x_10, 9); +x_27 = lean_ctor_get(x_10, 10); +x_28 = lean_ctor_get_uint8(x_10, sizeof(void*)*12); +x_29 = lean_ctor_get(x_10, 11); +x_30 = lean_ctor_get_uint8(x_10, sizeof(void*)*12 + 1); +lean_inc(x_29); +lean_inc(x_27); +lean_inc(x_26); +lean_inc(x_25); +lean_inc(x_24); +lean_inc(x_23); +lean_inc(x_22); +lean_inc(x_21); +lean_inc(x_20); +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_dec(x_10); +x_31 = l_Lean_replaceRef(x_1, x_22); +lean_dec(x_22); +x_32 = lean_alloc_ctor(0, 12, 2); +lean_ctor_set(x_32, 0, x_17); +lean_ctor_set(x_32, 1, x_18); +lean_ctor_set(x_32, 2, x_19); +lean_ctor_set(x_32, 3, x_20); +lean_ctor_set(x_32, 4, x_21); +lean_ctor_set(x_32, 5, x_31); +lean_ctor_set(x_32, 6, x_23); +lean_ctor_set(x_32, 7, x_24); +lean_ctor_set(x_32, 8, x_25); +lean_ctor_set(x_32, 9, x_26); +lean_ctor_set(x_32, 10, x_27); +lean_ctor_set(x_32, 11, x_29); +lean_ctor_set_uint8(x_32, sizeof(void*)*12, x_28); +lean_ctor_set_uint8(x_32, sizeof(void*)*12 + 1, x_30); +x_33 = l_Lean_Elab_Term_withAuxDecl___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_32, x_11, x_12); +return x_33; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withStructureLocalDecl___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_15; -x_15 = lean_usize_dec_eq(x_5, x_6); -if (x_15 == 0) -{ -lean_object* x_16; lean_object* x_17; -lean_dec(x_7); -x_16 = lean_array_uget(x_4, x_5); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); +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); -lean_inc(x_1); +x_11 = lean_ctor_get(x_10, 4); +lean_inc(x_11); +x_12 = lean_ctor_get(x_10, 3); +lean_inc(x_12); +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_17 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent(x_2, x_3, x_1, x_16, x_10, x_11, x_12, x_13, x_14); -if (lean_obj_tag(x_17) == 0) +lean_inc(x_1); +x_13 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkTypeFor(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_13) == 0) { -lean_object* x_18; lean_object* x_19; size_t x_20; size_t x_21; -x_18 = lean_ctor_get(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; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_13, 1); +lean_inc(x_15); +lean_dec(x_13); +x_16 = lean_ctor_get(x_1, 4); +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); -x_19 = lean_ctor_get(x_17, 1); +lean_dec(x_1); +x_19 = lean_ctor_get(x_10, 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_7 = x_18; -x_14 = x_19; -goto _start; +lean_dec(x_10); +x_20 = lean_apply_1(x_2, x_16); +x_21 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withStructureLocalDecl___rarg___lambda__1___boxed), 12, 5); +lean_closure_set(x_21, 0, x_19); +lean_closure_set(x_21, 1, x_12); +lean_closure_set(x_21, 2, x_14); +lean_closure_set(x_21, 3, x_11); +lean_closure_set(x_21, 4, x_20); +x_22 = l_Lean_Meta_withLCtx___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__3___rarg(x_17, x_18, x_21, x_3, x_4, x_5, x_6, x_7, x_8, x_15); +return x_22; } else { uint8_t x_23; -lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_23 = !lean_is_exclusive(x_17); +x_23 = !lean_is_exclusive(x_13); if (x_23 == 0) { -return x_17; +return x_13; } else { lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_17, 0); -x_25 = lean_ctor_get(x_17, 1); +x_24 = lean_ctor_get(x_13, 0); +x_25 = lean_ctor_get(x_13, 1); lean_inc(x_25); lean_inc(x_24); -lean_dec(x_17); +lean_dec(x_13); x_26 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_26, 0, x_24); lean_ctor_set(x_26, 1, x_25); @@ -30155,1803 +29188,1820 @@ return x_26; } } } -else +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withStructureLocalDecl(lean_object* x_1) { +_start: { -lean_object* x_27; -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_7); -lean_ctor_set(x_27, 1, x_14); -return x_27; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withStructureLocalDecl___rarg), 9, 0); +return x_2; +} } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withStructureLocalDecl___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; +x_13 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withStructureLocalDecl___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_1); +return x_13; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__9(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_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkInductiveType___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_12; -x_12 = lean_usize_dec_eq(x_2, x_3); -if (x_12 == 0) +uint8_t x_6; +x_6 = lean_expr_eqv(x_5, x_1); +if (x_6 == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_array_uget(x_1, x_2); -x_14 = lean_ctor_get(x_13, 2); -lean_inc(x_14); -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_Term_getFVarLocalDecl_x21(x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_14); -if (lean_obj_tag(x_15) == 0) +lean_object* x_7; +lean_dec(x_4); +x_7 = lean_box(0); +return x_7; +} +else { -lean_object* x_16; lean_object* x_17; uint8_t x_18; -x_16 = lean_ctor_get(x_15, 0); -lean_inc(x_16); -x_17 = lean_ctor_get(x_15, 1); -lean_inc(x_17); -lean_dec(x_15); -x_18 = l_Lean_Elab_Command_StructFieldInfo_isSubobject(x_13); -if (x_18 == 0) +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_8 = lean_unsigned_to_nat(0u); +x_9 = l_Array_extract___rarg(x_2, x_8, x_3); +x_10 = l_Lean_mkAppN(x_4, x_9); +lean_dec(x_9); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +return x_11; +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkInductiveType___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: { -size_t x_19; size_t x_20; -lean_dec(x_16); -lean_dec(x_13); -x_19 = 1; -x_20 = lean_usize_add(x_2, x_19); -x_2 = x_20; -x_11 = x_17; -goto _start; +lean_object* x_14; lean_object* x_15; uint8_t x_16; uint8_t x_17; uint8_t x_18; lean_object* x_19; +lean_inc(x_2); +x_14 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkInductiveType___lambda__1___boxed), 5, 4); +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); +x_15 = lean_replace_expr(x_14, x_5); +lean_dec(x_14); +x_16 = 0; +x_17 = 1; +x_18 = 1; +x_19 = l_Lean_Meta_mkForallFVars(x_2, x_15, x_16, x_17, x_18, 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; +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_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_20, x_7, x_8, x_9, x_10, x_11, x_12, x_21); +return x_22; } else { -uint8_t x_22; uint8_t x_23; -x_22 = l_Lean_LocalDecl_binderInfo(x_16); -lean_dec(x_16); -x_23 = l_Lean_BinderInfo_isInstImplicit(x_22); +uint8_t x_23; +x_23 = !lean_is_exclusive(x_19); if (x_23 == 0) { -size_t x_24; size_t x_25; -lean_dec(x_13); -x_24 = 1; -x_25 = lean_usize_add(x_2, x_24); -x_2 = x_25; -x_11 = x_17; -goto _start; +return x_19; } else { -lean_object* x_27; size_t x_28; size_t x_29; -x_27 = lean_array_push(x_4, x_13); -x_28 = 1; -x_29 = lean_usize_add(x_2, x_28); -x_2 = x_29; -x_4 = x_27; -x_11 = x_17; -goto _start; +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_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; +} +} +} +} +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkInductiveType___lambda__3___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Recursive structures are not yet supported.", 43, 43); +return x_1; } } +static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkInductiveType___lambda__3___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkInductiveType___lambda__3___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } -else +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkInductiveType___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_31; -lean_dec(x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -x_31 = !lean_is_exclusive(x_15); -if (x_31 == 0) +lean_object* x_14; uint8_t x_15; +x_14 = l_Lean_Expr_fvarId_x21(x_1); +x_15 = l_Lean_Expr_hasAnyFVar_visit___at_Lean_Expr_containsFVar___spec__1(x_14, x_6); +lean_dec(x_14); +if (x_15 == 0) { -return x_15; +lean_object* x_16; lean_object* x_17; +x_16 = lean_box(0); +x_17 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkInductiveType___lambda__2(x_1, x_5, x_2, x_3, x_6, x_16, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_11); +lean_dec(x_7); +return x_17; } else { -lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_32 = lean_ctor_get(x_15, 0); -x_33 = lean_ctor_get(x_15, 1); -lean_inc(x_33); -lean_inc(x_32); -lean_dec(x_15); -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_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_18 = lean_ctor_get(x_4, 0); +x_19 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkInductiveType___lambda__3___closed__2; +x_20 = l_Lean_throwErrorAt___at___private_Lean_Elab_Binders_0__Lean_Elab_Term_elabBinderViews_loop___spec__1(x_18, x_19, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +x_21 = !lean_is_exclusive(x_20); +if (x_21 == 0) +{ +return x_20; } else { -lean_object* x_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); -x_35 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_35, 0, x_4); -lean_ctor_set(x_35, 1, x_11); -return x_35; +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_20, 0); +x_23 = lean_ctor_get(x_20, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_20); +x_24 = lean_alloc_ctor(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_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__10(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkInductiveType(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, 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_5; -x_5 = lean_usize_dec_eq(x_2, x_3); -if (x_5 == 0) +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; +x_15 = lean_box(0); +x_16 = l_List_mapTR_loop___at_Lean_mkConstWithLevelParams___spec__1(x_3, x_15); +x_17 = lean_ctor_get(x_1, 4); +lean_inc(x_17); +lean_inc(x_17); +x_18 = l_Lean_Expr_const___override(x_17, x_16); +x_19 = !lean_is_exclusive(x_7); +if (x_19 == 0) { -lean_object* x_6; uint8_t x_7; size_t x_8; size_t x_9; -x_6 = lean_array_uget(x_1, x_2); -x_7 = l_Lean_Elab_Command_StructFieldInfo_isFromParent(x_6); -x_8 = 1; -x_9 = lean_usize_add(x_2, x_8); -if (x_7 == 0) +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_7, 0); +x_21 = lean_ctor_get(x_7, 1); +x_22 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_22, 0, x_5); +x_23 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkInductiveType___lambda__3___boxed), 13, 4); +lean_closure_set(x_23, 0, x_2); +lean_closure_set(x_23, 1, x_4); +lean_closure_set(x_23, 2, x_18); +lean_closure_set(x_23, 3, x_1); +x_24 = 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_25 = l_Lean_Meta_forallBoundedTelescope___at_Lean_Elab_Term_addAutoBoundImplicits_x27___spec__2___rarg(x_21, x_22, x_23, x_24, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +if (lean_obj_tag(x_25) == 0) { -lean_object* x_10; -x_10 = lean_array_push(x_4, x_6); -x_2 = x_9; -x_4 = x_10; -goto _start; +lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; +x_26 = lean_ctor_get(x_25, 0); +lean_inc(x_26); +x_27 = lean_ctor_get(x_25, 1); +lean_inc(x_27); +lean_dec(x_25); +x_28 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_6, x_8, x_9, x_10, x_11, x_12, x_13, x_27); +x_29 = !lean_is_exclusive(x_28); +if (x_29 == 0) +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; +x_30 = lean_ctor_get(x_28, 0); +x_31 = lean_ctor_get(x_28, 1); +x_32 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_26, x_8, x_9, x_10, x_11, x_12, x_13, x_31); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +x_33 = !lean_is_exclusive(x_32); +if (x_33 == 0) +{ +lean_object* x_34; lean_object* x_35; +x_34 = lean_ctor_get(x_32, 0); +lean_ctor_set(x_7, 1, x_34); +lean_ctor_set_tag(x_28, 1); +lean_ctor_set(x_28, 1, x_15); +lean_ctor_set(x_28, 0, x_7); +x_35 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_35, 0, x_17); +lean_ctor_set(x_35, 1, x_30); +lean_ctor_set(x_35, 2, x_28); +lean_ctor_set(x_32, 0, x_35); +return x_32; } else { -lean_dec(x_6); -x_2 = x_9; -goto _start; +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); +lean_ctor_set(x_7, 1, x_36); +lean_ctor_set_tag(x_28, 1); +lean_ctor_set(x_28, 1, x_15); +lean_ctor_set(x_28, 0, x_7); +x_38 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_38, 0, x_17); +lean_ctor_set(x_38, 1, x_30); +lean_ctor_set(x_38, 2, x_28); +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 { -return x_4; +lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_40 = lean_ctor_get(x_28, 0); +x_41 = lean_ctor_get(x_28, 1); +lean_inc(x_41); +lean_inc(x_40); +lean_dec(x_28); +x_42 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_26, x_8, x_9, x_10, x_11, x_12, x_13, x_41); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +x_43 = lean_ctor_get(x_42, 0); +lean_inc(x_43); +x_44 = lean_ctor_get(x_42, 1); +lean_inc(x_44); +if (lean_is_exclusive(x_42)) { + lean_ctor_release(x_42, 0); + lean_ctor_release(x_42, 1); + x_45 = x_42; +} else { + lean_dec_ref(x_42); + x_45 = lean_box(0); } +lean_ctor_set(x_7, 1, x_43); +x_46 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_46, 0, x_7); +lean_ctor_set(x_46, 1, x_15); +x_47 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_47, 0, x_17); +lean_ctor_set(x_47, 1, x_40); +lean_ctor_set(x_47, 2, x_46); +if (lean_is_scalar(x_45)) { + x_48 = lean_alloc_ctor(0, 2, 0); +} else { + x_48 = x_45; +} +lean_ctor_set(x_48, 0, x_47); +lean_ctor_set(x_48, 1, x_44); +return x_48; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__11___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_10 = lean_ctor_get(x_1, 2); -lean_inc(x_10); -x_11 = lean_ctor_get(x_1, 0); -lean_inc(x_11); -lean_dec(x_1); -x_12 = l_Lean_Elab_addAuxDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__18(x_10, x_11, x_11, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +uint8_t x_49; +lean_free_object(x_7); +lean_dec(x_20); +lean_dec(x_17); +lean_dec(x_13); +lean_dec(x_12); lean_dec(x_11); -return x_12; -} -} -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__11___closed__1() { -_start: +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +x_49 = !lean_is_exclusive(x_25); +if (x_49 == 0) { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("', it is equal to structure constructor name", 44, 44); -return x_1; -} +return x_25; } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__11___closed__2() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__11___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_50 = lean_ctor_get(x_25, 0); +x_51 = lean_ctor_get(x_25, 1); +lean_inc(x_51); +lean_inc(x_50); +lean_dec(x_25); +x_52 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_52, 0, x_50); +lean_ctor_set(x_52, 1, x_51); +return x_52; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__11(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_eq(x_3, x_4); -if (x_13 == 0) -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; -lean_dec(x_5); -x_14 = lean_array_uget(x_2, x_3); -x_15 = lean_ctor_get(x_14, 2); -lean_inc(x_15); -x_16 = lean_ctor_get(x_1, 9); -x_17 = lean_ctor_get(x_16, 3); -x_18 = lean_name_eq(x_15, x_17); -lean_dec(x_15); -if (x_18 == 0) -{ -lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; size_t x_23; size_t x_24; -x_19 = lean_box(0); -lean_inc(x_10); -x_20 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__11___lambda__1(x_14, x_19, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_20, 1); -lean_inc(x_22); -lean_dec(x_20); -x_23 = 1; -x_24 = lean_usize_add(x_3, x_23); -x_3 = x_24; -x_5 = x_21; -x_12 = x_22; -goto _start; } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; -x_26 = lean_ctor_get(x_14, 0); -lean_inc(x_26); -x_27 = lean_ctor_get(x_14, 3); -lean_inc(x_27); -lean_dec(x_14); -x_28 = l_Lean_MessageData_ofName(x_27); -x_29 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___closed__2; -x_30 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_30, 0, x_29); -lean_ctor_set(x_30, 1, x_28); -x_31 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__11___closed__2; -x_32 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_32, 0, x_30); -lean_ctor_set(x_32, 1, x_31); -x_33 = l_Lean_throwErrorAt___at___private_Lean_Elab_Binders_0__Lean_Elab_Term_elabBinderViews_loop___spec__1(x_26, x_32, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_26); -x_34 = !lean_is_exclusive(x_33); -if (x_34 == 0) +lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; uint8_t x_57; lean_object* x_58; +x_53 = lean_ctor_get(x_7, 0); +x_54 = lean_ctor_get(x_7, 1); +lean_inc(x_54); +lean_inc(x_53); +lean_dec(x_7); +x_55 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_55, 0, x_5); +x_56 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkInductiveType___lambda__3___boxed), 13, 4); +lean_closure_set(x_56, 0, x_2); +lean_closure_set(x_56, 1, x_4); +lean_closure_set(x_56, 2, x_18); +lean_closure_set(x_56, 3, x_1); +x_57 = 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_58 = l_Lean_Meta_forallBoundedTelescope___at_Lean_Elab_Term_addAutoBoundImplicits_x27___spec__2___rarg(x_54, x_55, x_56, x_57, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +if (lean_obj_tag(x_58) == 0) { -return x_33; +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_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_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_6, x_8, x_9, x_10, x_11, x_12, x_13, 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); +if (lean_is_exclusive(x_61)) { + lean_ctor_release(x_61, 0); + lean_ctor_release(x_61, 1); + x_64 = x_61; +} else { + lean_dec_ref(x_61); + x_64 = lean_box(0); +} +x_65 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_59, x_8, x_9, x_10, x_11, x_12, x_13, x_63); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +x_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; +} else { + lean_dec_ref(x_65); + x_68 = lean_box(0); } -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_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; +x_69 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_69, 0, x_53); +lean_ctor_set(x_69, 1, x_66); +if (lean_is_scalar(x_64)) { + x_70 = lean_alloc_ctor(1, 2, 0); +} else { + x_70 = x_64; + lean_ctor_set_tag(x_70, 1); } +lean_ctor_set(x_70, 0, x_69); +lean_ctor_set(x_70, 1, x_15); +x_71 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_71, 0, x_17); +lean_ctor_set(x_71, 1, x_62); +lean_ctor_set(x_71, 2, x_70); +if (lean_is_scalar(x_68)) { + x_72 = lean_alloc_ctor(0, 2, 0); +} else { + x_72 = x_68; } +lean_ctor_set(x_72, 0, x_71); +lean_ctor_set(x_72, 1, x_67); +return x_72; } else { -lean_object* x_38; +lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; +lean_dec(x_53); +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_6); -x_38 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_38, 0, x_5); -lean_ctor_set(x_38, 1, x_12); -return x_38; +x_73 = lean_ctor_get(x_58, 0); +lean_inc(x_73); +x_74 = lean_ctor_get(x_58, 1); +lean_inc(x_74); +if (lean_is_exclusive(x_58)) { + lean_ctor_release(x_58, 0); + lean_ctor_release(x_58, 1); + x_75 = x_58; +} else { + lean_dec_ref(x_58); + 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; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___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: -{ -size_t x_10; size_t x_11; lean_object* x_12; lean_object* x_13; -x_10 = lean_array_size(x_1); -x_11 = 0; -x_12 = lean_box(0); -x_13 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__2(x_1, x_10, x_11, x_12, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_13) == 0) -{ -uint8_t x_14; -x_14 = !lean_is_exclusive(x_13); -if (x_14 == 0) -{ -lean_object* x_15; -x_15 = lean_ctor_get(x_13, 0); -lean_dec(x_15); -lean_ctor_set(x_13, 0, x_12); -return x_13; } -else -{ -lean_object* x_16; lean_object* x_17; -x_16 = lean_ctor_get(x_13, 1); -lean_inc(x_16); -lean_dec(x_13); -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_12); -lean_ctor_set(x_17, 1, x_16); -return x_17; } } -else -{ -uint8_t x_18; -x_18 = !lean_is_exclusive(x_13); -if (x_18 == 0) +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkInductiveType___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: { -return x_13; +lean_object* x_6; +x_6 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkInductiveType___lambda__1(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_6; } -else +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkInductiveType___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: { -lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_19 = lean_ctor_get(x_13, 0); -x_20 = lean_ctor_get(x_13, 1); -lean_inc(x_20); -lean_inc(x_19); -lean_dec(x_13); -x_21 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_21, 0, x_19); -lean_ctor_set(x_21, 1, x_20); -return x_21; +lean_object* x_14; +x_14 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkInductiveType___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); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +return x_14; } } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkInductiveType___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; +x_14 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkInductiveType___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_12); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_4); +return x_14; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_mkStructureDecl___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: { -lean_object* x_12; -lean_inc(x_5); -x_12 = l_Lean_mkConstWithLevelParams___at_Lean_Elab_Term_expandDeclId___spec__7(x_1, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_12) == 0) +uint8_t x_12; +x_12 = lean_usize_dec_lt(x_3, 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_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_unsigned_to_nat(1u); -x_16 = l_Lean_Syntax_getArg(x_2, x_15); -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_17 = l_Lean_Elab_Term_addLocalVarInfo(x_16, x_13, x_5, x_6, x_7, x_8, x_9, x_10, x_14); -if (lean_obj_tag(x_17) == 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_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; lean_object* x_22; -x_18 = lean_ctor_get(x_17, 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; uint8_t x_20; +lean_dec(x_4); +x_14 = lean_array_uget(x_1, x_3); +x_15 = lean_st_ref_get(x_10, x_11); +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_15, 1); +lean_inc(x_17); +lean_dec(x_15); +x_18 = lean_ctor_get(x_16, 0); lean_inc(x_18); -lean_dec(x_17); -x_19 = lean_ctor_get(x_4, 9); +lean_dec(x_16); +x_19 = lean_ctor_get(x_14, 2); lean_inc(x_19); -lean_dec(x_4); -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); -x_21 = 1; -x_22 = l_Lean_Syntax_getPos_x3f(x_20, x_21); -if (lean_obj_tag(x_22) == 0) +x_20 = l_Lean_Environment_contains(x_18, x_19); +if (x_20 == 0) { -lean_object* x_23; lean_object* x_24; -lean_dec(x_20); +size_t x_21; size_t x_22; lean_object* x_23; lean_dec(x_19); +lean_dec(x_14); +x_21 = 1; +x_22 = lean_usize_add(x_3, x_21); x_23 = lean_box(0); -x_24 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__1(x_3, x_23, x_5, x_6, x_7, x_8, x_9, x_10, x_18); -return x_24; +x_3 = x_22; +x_4 = x_23; +x_11 = x_17; +goto _start; } else { -lean_object* x_25; lean_object* x_26; -lean_dec(x_22); -x_25 = lean_ctor_get(x_19, 3); -lean_inc(x_25); -lean_dec(x_19); +lean_object* x_25; lean_inc(x_5); -x_26 = l_Lean_mkConstWithLevelParams___at_Lean_Elab_Term_expandDeclId___spec__7(x_25, x_5, x_6, x_7, x_8, x_9, x_10, x_18); -if (lean_obj_tag(x_26) == 0) +x_25 = l_Lean_mkConstWithLevelParams___at_Lean_Elab_Term_expandDeclId___spec__7(x_19, x_5, x_6, x_7, x_8, x_9, x_10, x_17); +if (lean_obj_tag(x_25) == 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_26, 0); +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_26 = lean_ctor_get(x_25, 0); +lean_inc(x_26); +x_27 = lean_ctor_get(x_25, 1); lean_inc(x_27); -x_28 = lean_ctor_get(x_26, 1); +lean_dec(x_25); +x_28 = lean_ctor_get(x_14, 0); lean_inc(x_28); -lean_dec(x_26); +lean_dec(x_14); x_29 = lean_box(0); x_30 = lean_box(0); +x_31 = 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_31 = l_Lean_Elab_Term_addTermInfo_x27(x_20, x_27, x_29, x_29, x_30, x_21, x_5, x_6, x_7, x_8, x_9, x_10, x_28); -if (lean_obj_tag(x_31) == 0) +x_32 = l_Lean_Elab_Term_addTermInfo_x27(x_28, x_26, x_29, x_29, x_30, x_31, x_5, x_6, x_7, x_8, x_9, x_10, x_27); +if (lean_obj_tag(x_32) == 0) { -lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_32 = lean_ctor_get(x_31, 0); -lean_inc(x_32); -x_33 = lean_ctor_get(x_31, 1); +lean_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_31); -x_34 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__1(x_3, x_32, x_5, x_6, x_7, x_8, x_9, x_10, x_33); lean_dec(x_32); -return x_34; -} -else -{ -uint8_t x_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); -x_35 = !lean_is_exclusive(x_31); -if (x_35 == 0) -{ -return x_31; -} -else -{ -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; -} -} +x_34 = 1; +x_35 = lean_usize_add(x_3, x_34); +x_36 = lean_box(0); +x_3 = x_35; +x_4 = x_36; +x_11 = x_33; +goto _start; } else { -uint8_t x_39; -lean_dec(x_20); +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_39 = !lean_is_exclusive(x_26); -if (x_39 == 0) +x_38 = !lean_is_exclusive(x_32); +if (x_38 == 0) { -return x_26; +return x_32; } else { -lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_40 = lean_ctor_get(x_26, 0); -x_41 = lean_ctor_get(x_26, 1); -lean_inc(x_41); +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_dec(x_26); -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_inc(x_39); +lean_dec(x_32); +x_41 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_41, 0, x_39); +lean_ctor_set(x_41, 1, x_40); +return x_41; } } } else { -uint8_t x_43; +uint8_t x_42; +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_43 = !lean_is_exclusive(x_17); -if (x_43 == 0) +x_42 = !lean_is_exclusive(x_25); +if (x_42 == 0) { -return x_17; +return x_25; } else { -lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_44 = lean_ctor_get(x_17, 0); -x_45 = lean_ctor_get(x_17, 1); -lean_inc(x_45); +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_25, 0); +x_44 = lean_ctor_get(x_25, 1); lean_inc(x_44); -lean_dec(x_17); -x_46 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_46, 0, x_44); -lean_ctor_set(x_46, 1, x_45); -return x_46; +lean_inc(x_43); +lean_dec(x_25); +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_EXPORT lean_object* l_List_forM___at_Lean_Elab_Command_mkStructureDecl___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: { -uint8_t x_47; -lean_dec(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; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_47 = !lean_is_exclusive(x_12); -if (x_47 == 0) +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; +} +else { -return x_12; +lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; lean_object* 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); +lean_dec(x_1); +x_13 = 0; +x_14 = lean_unsigned_to_nat(1000u); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_15 = l_Lean_Meta_addInstance(x_11, x_13, x_14, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_15) == 0) +{ +lean_object* x_16; +x_16 = lean_ctor_get(x_15, 1); +lean_inc(x_16); +lean_dec(x_15); +x_1 = x_12; +x_8 = x_16; +goto _start; } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_ctor_get(x_12, 0); -x_49 = lean_ctor_get(x_12, 1); -lean_inc(x_49); -lean_inc(x_48); +uint8_t x_18; lean_dec(x_12); -x_50 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_50, 0, x_48); -lean_ctor_set(x_50, 1, x_49); -return x_50; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_18 = !lean_is_exclusive(x_15); +if (x_18 == 0) +{ +return x_15; } +else +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; +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(1, 2, 0); +lean_ctor_set(x_21, 0, x_19); +lean_ctor_set(x_21, 1, x_20); +return x_21; } } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__3___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_withSaveInfoContext___at___private_Lean_Elab_PreDefinition_Basic_0__Lean_Elab_addNonRecAux___spec__1___lambda__1___boxed), 7, 0); -return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_mkStructureDecl___spec__3(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { -lean_object* x_17; -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_1); -x_17 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectLevelParamsInStructure(x_1, x_2, x_3, x_4, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_17) == 0) -{ -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -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_5, 2); -lean_inc(x_20); -x_21 = lean_ctor_get(x_5, 3); -lean_inc(x_21); -x_22 = l_Lean_Elab_sortDeclLevelParams(x_20, x_21, x_18); -if (lean_obj_tag(x_22) == 0) -{ -uint8_t x_23; -lean_dec(x_7); -lean_dec(x_5); -lean_dec(x_2); -lean_dec(x_1); -x_23 = !lean_is_exclusive(x_22); -if (x_23 == 0) +uint8_t x_5; +x_5 = lean_usize_dec_eq(x_2, x_3); +if (x_5 == 0) { -lean_object* x_24; uint8_t x_25; -lean_ctor_set_tag(x_22, 3); -x_24 = l_Lean_MessageData_ofFormat(x_22); -x_25 = !lean_is_exclusive(x_14); -if (x_25 == 0) +lean_object* x_6; uint8_t x_7; size_t x_8; size_t x_9; +x_6 = lean_array_uget(x_1, x_2); +x_7 = l_Lean_Elab_Command_StructFieldInfo_isFromParent(x_6); +x_8 = 1; +x_9 = lean_usize_add(x_2, x_8); +if (x_7 == 0) { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_14, 5); -x_27 = l_Lean_replaceRef(x_6, x_26); -lean_dec(x_26); +lean_object* x_10; lean_object* x_11; uint8_t x_12; lean_object* x_13; +x_10 = lean_ctor_get(x_6, 3); +lean_inc(x_10); lean_dec(x_6); -lean_ctor_set(x_14, 5, x_27); -x_28 = l_Lean_throwError___at_Lean_Elab_Term_throwErrorIfErrors___spec__1(x_24, x_10, x_11, x_12, x_13, x_14, x_15, x_19); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -return x_28; +x_11 = l_Lean_Expr_fvarId_x21(x_10); +lean_dec(x_10); +x_12 = 0; +x_13 = l_Lean_LocalContext_setBinderInfo(x_4, x_11, x_12); +x_2 = x_9; +x_4 = x_13; +goto _start; } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; 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; uint8_t x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; -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); -x_35 = lean_ctor_get(x_14, 6); -x_36 = lean_ctor_get(x_14, 7); -x_37 = lean_ctor_get(x_14, 8); -x_38 = lean_ctor_get(x_14, 9); -x_39 = lean_ctor_get(x_14, 10); -x_40 = lean_ctor_get_uint8(x_14, sizeof(void*)*12); -x_41 = lean_ctor_get(x_14, 11); -x_42 = lean_ctor_get_uint8(x_14, sizeof(void*)*12 + 1); -lean_inc(x_41); -lean_inc(x_39); -lean_inc(x_38); -lean_inc(x_37); -lean_inc(x_36); -lean_inc(x_35); -lean_inc(x_34); -lean_inc(x_33); -lean_inc(x_32); -lean_inc(x_31); -lean_inc(x_30); -lean_inc(x_29); -lean_dec(x_14); -x_43 = l_Lean_replaceRef(x_6, x_34); -lean_dec(x_34); lean_dec(x_6); -x_44 = lean_alloc_ctor(0, 12, 2); -lean_ctor_set(x_44, 0, x_29); -lean_ctor_set(x_44, 1, x_30); -lean_ctor_set(x_44, 2, x_31); -lean_ctor_set(x_44, 3, x_32); -lean_ctor_set(x_44, 4, x_33); -lean_ctor_set(x_44, 5, x_43); -lean_ctor_set(x_44, 6, x_35); -lean_ctor_set(x_44, 7, x_36); -lean_ctor_set(x_44, 8, x_37); -lean_ctor_set(x_44, 9, x_38); -lean_ctor_set(x_44, 10, x_39); -lean_ctor_set(x_44, 11, x_41); -lean_ctor_set_uint8(x_44, sizeof(void*)*12, x_40); -lean_ctor_set_uint8(x_44, sizeof(void*)*12 + 1, x_42); -x_45 = l_Lean_throwError___at_Lean_Elab_Term_throwErrorIfErrors___spec__1(x_24, x_10, x_11, x_12, x_13, x_44, x_15, x_19); -lean_dec(x_15); -lean_dec(x_44); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -return x_45; +x_2 = x_9; +goto _start; } } 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; uint8_t 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; -x_46 = lean_ctor_get(x_22, 0); -lean_inc(x_46); -lean_dec(x_22); -x_47 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_47, 0, x_46); -x_48 = l_Lean_MessageData_ofFormat(x_47); -x_49 = lean_ctor_get(x_14, 0); -lean_inc(x_49); -x_50 = lean_ctor_get(x_14, 1); -lean_inc(x_50); -x_51 = lean_ctor_get(x_14, 2); -lean_inc(x_51); -x_52 = lean_ctor_get(x_14, 3); -lean_inc(x_52); -x_53 = lean_ctor_get(x_14, 4); -lean_inc(x_53); -x_54 = lean_ctor_get(x_14, 5); -lean_inc(x_54); -x_55 = lean_ctor_get(x_14, 6); -lean_inc(x_55); -x_56 = lean_ctor_get(x_14, 7); -lean_inc(x_56); -x_57 = lean_ctor_get(x_14, 8); -lean_inc(x_57); -x_58 = lean_ctor_get(x_14, 9); -lean_inc(x_58); -x_59 = lean_ctor_get(x_14, 10); -lean_inc(x_59); -x_60 = lean_ctor_get_uint8(x_14, sizeof(void*)*12); -x_61 = lean_ctor_get(x_14, 11); -lean_inc(x_61); -x_62 = lean_ctor_get_uint8(x_14, sizeof(void*)*12 + 1); -if (lean_is_exclusive(x_14)) { - lean_ctor_release(x_14, 0); - lean_ctor_release(x_14, 1); - lean_ctor_release(x_14, 2); - lean_ctor_release(x_14, 3); - lean_ctor_release(x_14, 4); - lean_ctor_release(x_14, 5); - lean_ctor_release(x_14, 6); - lean_ctor_release(x_14, 7); - lean_ctor_release(x_14, 8); - lean_ctor_release(x_14, 9); - lean_ctor_release(x_14, 10); - lean_ctor_release(x_14, 11); - x_63 = x_14; -} else { - lean_dec_ref(x_14); - x_63 = lean_box(0); +return x_4; } -x_64 = l_Lean_replaceRef(x_6, x_54); -lean_dec(x_54); +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_mkStructureDecl___spec__4(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; uint8_t x_7; size_t x_8; size_t x_9; +x_6 = lean_array_uget(x_1, x_2); +x_7 = l_Lean_Expr_isFVar(x_6); +x_8 = 1; +x_9 = lean_usize_add(x_2, x_8); +if (x_7 == 0) +{ +lean_dec(x_6); +x_2 = x_9; +goto _start; +} +else +{ +lean_object* x_11; uint8_t x_12; lean_object* x_13; +x_11 = l_Lean_Expr_fvarId_x21(x_6); lean_dec(x_6); -if (lean_is_scalar(x_63)) { - x_65 = lean_alloc_ctor(0, 12, 2); -} else { - x_65 = x_63; -} -lean_ctor_set(x_65, 0, x_49); -lean_ctor_set(x_65, 1, x_50); -lean_ctor_set(x_65, 2, x_51); -lean_ctor_set(x_65, 3, x_52); -lean_ctor_set(x_65, 4, x_53); -lean_ctor_set(x_65, 5, x_64); -lean_ctor_set(x_65, 6, x_55); -lean_ctor_set(x_65, 7, x_56); -lean_ctor_set(x_65, 8, x_57); -lean_ctor_set(x_65, 9, x_58); -lean_ctor_set(x_65, 10, x_59); -lean_ctor_set(x_65, 11, x_61); -lean_ctor_set_uint8(x_65, sizeof(void*)*12, x_60); -lean_ctor_set_uint8(x_65, sizeof(void*)*12 + 1, x_62); -x_66 = l_Lean_throwError___at_Lean_Elab_Term_throwErrorIfErrors___spec__1(x_48, x_10, x_11, x_12, x_13, x_65, x_15, x_19); -lean_dec(x_15); -lean_dec(x_65); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -return x_66; +x_12 = 1; +x_13 = l_Lean_LocalContext_setBinderInfo(x_4, x_11, x_12); +x_2 = x_9; +x_4 = x_13; +goto _start; } } else { -lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_67 = lean_ctor_get(x_22, 0); -lean_inc(x_67); -lean_dec(x_22); -x_68 = l_Array_append___rarg(x_2, x_3); -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_68); -lean_inc(x_67); -lean_inc(x_5); -x_69 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCtor(x_5, x_67, x_68, x_4, x_10, x_11, x_12, x_13, x_14, x_15, x_19); -if (lean_obj_tag(x_69) == 0) +return x_4; +} +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_mkStructureDecl___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, 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_70; lean_object* x_71; uint8_t x_72; uint8_t x_73; uint8_t x_74; lean_object* x_75; -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 = 0; -x_73 = 1; -x_74 = 1; -lean_inc(x_68); -x_75 = l_Lean_Meta_mkForallFVars(x_68, x_1, x_72, x_73, x_74, x_12, x_13, x_14, x_15, x_71); -if (lean_obj_tag(x_75) == 0) +uint8_t x_15; +x_15 = lean_usize_dec_eq(x_5, x_6); +if (x_15 == 0) { -lean_object* x_76; lean_object* x_77; lean_object* x_78; uint8_t x_79; -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_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_76, x_10, x_11, x_12, x_13, x_14, x_15, x_77); -x_79 = !lean_is_exclusive(x_78); -if (x_79 == 0) +lean_object* x_16; uint8_t x_17; +lean_dec(x_7); +x_16 = lean_array_uget(x_4, x_5); +x_17 = lean_ctor_get_uint8(x_16, sizeof(void*)*4); +if (x_17 == 0) { -lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; uint8_t x_88; lean_object* x_89; lean_object* x_90; -x_80 = lean_ctor_get(x_78, 0); -x_81 = lean_ctor_get(x_78, 1); -x_82 = lean_ctor_get(x_5, 4); -lean_inc(x_82); -x_83 = lean_box(0); -lean_ctor_set_tag(x_78, 1); -lean_ctor_set(x_78, 1, x_83); -lean_ctor_set(x_78, 0, x_70); -lean_inc(x_82); -x_84 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_84, 0, x_82); -lean_ctor_set(x_84, 1, x_80); -lean_ctor_set(x_84, 2, x_78); -x_85 = lean_array_get_size(x_68); -x_86 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_86, 0, x_84); -lean_ctor_set(x_86, 1, x_83); -x_87 = lean_ctor_get(x_5, 1); -lean_inc(x_87); -x_88 = lean_ctor_get_uint8(x_87, sizeof(void*)*2 + 3); -lean_inc(x_85); -lean_inc(x_67); -x_89 = lean_alloc_ctor(6, 3, 1); -lean_ctor_set(x_89, 0, x_67); -lean_ctor_set(x_89, 1, x_85); -lean_ctor_set(x_89, 2, x_86); -lean_ctor_set_uint8(x_89, sizeof(void*)*3, x_88); -lean_inc(x_15); -lean_inc(x_14); +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_16, 2); +lean_inc(x_18); +x_19 = lean_ctor_get(x_16, 3); +lean_inc(x_19); +lean_dec(x_16); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); -lean_inc(x_89); -x_90 = l_Lean_Elab_Term_ensureNoUnassignedMVars(x_89, x_10, x_11, x_12, x_13, x_14, x_15, x_81); -if (lean_obj_tag(x_90) == 0) +lean_inc(x_1); +lean_inc(x_3); +lean_inc(x_2); +x_20 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent(x_2, x_3, x_1, x_18, x_19, x_10, x_11, x_12, x_13, x_14); +if (lean_obj_tag(x_20) == 0) { -lean_object* x_91; lean_object* x_92; -x_91 = lean_ctor_get(x_90, 1); -lean_inc(x_91); -lean_dec(x_90); -lean_inc(x_15); -lean_inc(x_14); -x_92 = l_Lean_addDecl(x_89, x_14, x_15, x_91); -if (lean_obj_tag(x_92) == 0) +lean_object* x_21; lean_object* x_22; size_t x_23; size_t x_24; +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +x_23 = 1; +x_24 = lean_usize_add(x_5, x_23); +x_5 = x_24; +x_7 = x_21; +x_14 = x_22; +goto _start; +} +else { -lean_object* x_93; lean_object* x_94; lean_object* x_95; uint8_t x_96; uint8_t x_97; lean_object* x_98; -x_93 = lean_ctor_get(x_92, 1); -lean_inc(x_93); -lean_dec(x_92); -x_94 = lean_array_get_size(x_4); -x_95 = lean_unsigned_to_nat(0u); -x_96 = lean_nat_dec_lt(x_95, x_94); -x_97 = lean_ctor_get_uint8(x_5, sizeof(void*)*11); -if (x_96 == 0) +uint8_t x_26; +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_26 = !lean_is_exclusive(x_20); +if (x_26 == 0) { -lean_object* x_214; -x_214 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; -x_98 = x_214; -goto block_213; +return x_20; } else { -uint8_t x_215; -x_215 = lean_nat_dec_le(x_94, x_94); -if (x_215 == 0) +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_dec(x_20); +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_27); +lean_ctor_set(x_29, 1, x_28); +return x_29; +} +} +} +else { -lean_object* x_216; -x_216 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; -x_98 = x_216; -goto block_213; +size_t x_30; size_t x_31; lean_object* x_32; +lean_dec(x_16); +x_30 = 1; +x_31 = lean_usize_add(x_5, x_30); +x_32 = lean_box(0); +x_5 = x_31; +x_7 = x_32; +goto _start; +} } else { -size_t x_217; size_t x_218; lean_object* x_219; lean_object* x_220; -x_217 = 0; -x_218 = lean_usize_of_nat(x_94); -x_219 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; -x_220 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__10(x_4, x_217, x_218, x_219); -x_98 = x_220; -goto block_213; +lean_object* x_34; +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_34 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_34, 0, x_7); +lean_ctor_set(x_34, 1, x_14); +return x_34; } } -block_213: +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_mkStructureDecl___spec__6(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +uint8_t x_12; +x_12 = lean_usize_dec_eq(x_2, x_3); +if (x_12 == 0) { -lean_object* x_99; lean_object* x_100; lean_object* x_101; -x_99 = lean_array_to_list(x_98); -x_100 = l_List_mapTR_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__1(x_99, x_83); +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_array_uget(x_1, x_2); +x_14 = lean_ctor_get(x_13, 3); lean_inc(x_14); lean_inc(x_10); -lean_inc(x_82); -x_101 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections(x_82, x_100, x_97, x_10, x_11, x_12, x_13, x_14, x_15, x_93); -if (lean_obj_tag(x_101) == 0) +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_Term_getFVarLocalDecl_x21(x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_14); +if (lean_obj_tag(x_15) == 0) { -lean_object* x_102; lean_object* x_103; -x_102 = lean_ctor_get(x_101, 1); -lean_inc(x_102); -lean_dec(x_101); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_82); -x_103 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure(x_82, x_4, x_10, x_11, x_12, x_13, x_14, x_15, x_102); -if (lean_obj_tag(x_103) == 0) +lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_15, 1); +lean_inc(x_17); +lean_dec(x_15); +x_18 = l_Lean_Elab_Command_StructFieldInfo_isSubobject(x_13); +if (x_18 == 0) { -lean_object* x_104; lean_object* x_105; -x_104 = lean_ctor_get(x_103, 1); -lean_inc(x_104); -lean_dec(x_103); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_82); -x_105 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions(x_82, x_10, x_11, x_12, x_13, x_14, x_15, x_104); -if (lean_obj_tag(x_105) == 0) +size_t x_19; size_t x_20; +lean_dec(x_16); +lean_dec(x_13); +x_19 = 1; +x_20 = lean_usize_add(x_2, x_19); +x_2 = x_20; +x_11 = x_17; +goto _start; +} +else { -lean_object* x_106; lean_object* x_107; lean_object* x_108; -x_106 = lean_ctor_get(x_105, 1); -lean_inc(x_106); -lean_dec(x_105); -if (x_96 == 0) +uint8_t x_22; uint8_t x_23; +x_22 = l_Lean_LocalDecl_binderInfo(x_16); +lean_dec(x_16); +x_23 = l_Lean_BinderInfo_isInstImplicit(x_22); +if (x_23 == 0) { -lean_object* x_188; -x_188 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; -x_107 = x_188; -x_108 = x_106; -goto block_187; +size_t x_24; size_t x_25; +lean_dec(x_13); +x_24 = 1; +x_25 = lean_usize_add(x_2, x_24); +x_2 = x_25; +x_11 = x_17; +goto _start; } else { -uint8_t x_189; -x_189 = lean_nat_dec_le(x_94, x_94); -if (x_189 == 0) -{ -lean_object* x_190; -x_190 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; -x_107 = x_190; -x_108 = x_106; -goto block_187; +lean_object* x_27; size_t x_28; size_t x_29; +x_27 = lean_array_push(x_4, x_13); +x_28 = 1; +x_29 = lean_usize_add(x_2, x_28); +x_2 = x_29; +x_4 = x_27; +x_11 = x_17; +goto _start; +} +} } else { -size_t x_191; size_t x_192; lean_object* x_193; lean_object* x_194; -x_191 = 0; -x_192 = lean_usize_of_nat(x_94); -x_193 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; -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_194 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__9(x_4, x_191, x_192, x_193, x_10, x_11, x_12, x_13, x_14, x_15, x_106); -if (lean_obj_tag(x_194) == 0) +uint8_t x_31; +lean_dec(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_31 = !lean_is_exclusive(x_15); +if (x_31 == 0) { -lean_object* x_195; lean_object* x_196; -x_195 = lean_ctor_get(x_194, 0); -lean_inc(x_195); -x_196 = lean_ctor_get(x_194, 1); -lean_inc(x_196); -lean_dec(x_194); -x_107 = x_195; -x_108 = x_196; -goto block_187; +return x_15; } else { -uint8_t x_197; -lean_dec(x_94); -lean_dec(x_87); -lean_dec(x_85); -lean_dec(x_82); -lean_dec(x_68); -lean_dec(x_67); +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_15, 0); +x_33 = lean_ctor_get(x_15, 1); +lean_inc(x_33); +lean_inc(x_32); lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); +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_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); -x_197 = !lean_is_exclusive(x_194); -if (x_197 == 0) -{ -return x_194; -} -else -{ -lean_object* x_198; lean_object* x_199; lean_object* x_200; -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_alloc_ctor(1, 2, 0); -lean_ctor_set(x_200, 0, x_198); -lean_ctor_set(x_200, 1, x_199); -return x_200; -} +x_35 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_35, 0, x_4); +lean_ctor_set(x_35, 1, x_11); +return x_35; } } } -block_187: -{ -lean_object* x_109; lean_object* x_110; lean_object* x_111; -lean_inc(x_5); -lean_inc(x_82); -x_109 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__2___boxed), 11, 4); -lean_closure_set(x_109, 0, x_82); -lean_closure_set(x_109, 1, x_6); -lean_closure_set(x_109, 2, x_7); -lean_closure_set(x_109, 3, x_5); -x_110 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__3___closed__1; -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_111 = l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at___private_Lean_Elab_PreDefinition_Basic_0__Lean_Elab_addNonRecAux___spec__2(x_109, x_110, x_10, x_11, x_12, x_13, x_14, x_15, x_108); -if (lean_obj_tag(x_111) == 0) -{ -lean_object* x_112; lean_object* x_113; uint8_t x_114; lean_object* x_115; -x_112 = lean_ctor_get(x_111, 1); -lean_inc(x_112); -lean_dec(x_111); -x_113 = lean_ctor_get(x_87, 1); -lean_inc(x_113); -lean_dec(x_87); -x_114 = 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_115 = l_Lean_Elab_Term_applyAttributesAt(x_82, x_113, x_114, x_10, x_11, x_12, x_13, x_14, x_15, x_112); -if (lean_obj_tag(x_115) == 0) +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___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_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; -x_116 = lean_ctor_get(x_115, 1); -lean_inc(x_116); -lean_dec(x_115); -x_117 = lean_array_to_list(x_107); -x_118 = l_List_mapTR_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__1(x_117, x_83); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -x_119 = l_List_forM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__3(x_118, x_10, x_11, x_12, x_13, x_14, x_15, x_116); -if (lean_obj_tag(x_119) == 0) +size_t x_10; size_t x_11; lean_object* x_12; lean_object* x_13; +x_10 = lean_array_size(x_1); +x_11 = 0; +x_12 = lean_box(0); +x_13 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_mkStructureDecl___spec__1(x_1, x_10, x_11, x_12, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_13) == 0) { -lean_object* x_120; lean_object* x_121; uint8_t x_122; lean_object* x_123; -x_120 = lean_ctor_get(x_119, 1); -lean_inc(x_120); -lean_dec(x_119); -x_121 = lean_array_get_size(x_8); -x_122 = lean_nat_dec_lt(x_95, x_121); -if (x_122 == 0) +uint8_t x_14; +x_14 = !lean_is_exclusive(x_13); +if (x_14 == 0) { -lean_dec(x_121); -lean_dec(x_67); -lean_dec(x_5); -x_123 = x_120; -goto block_164; +lean_object* x_15; +x_15 = lean_ctor_get(x_13, 0); +lean_dec(x_15); +lean_ctor_set(x_13, 0, x_12); +return x_13; } else { -uint8_t x_165; -x_165 = lean_nat_dec_le(x_121, x_121); -if (x_165 == 0) -{ -lean_dec(x_121); -lean_dec(x_67); -lean_dec(x_5); -x_123 = x_120; -goto block_164; +lean_object* x_16; lean_object* x_17; +x_16 = lean_ctor_get(x_13, 1); +lean_inc(x_16); +lean_dec(x_13); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_12); +lean_ctor_set(x_17, 1, x_16); +return x_17; } -else -{ -size_t x_166; size_t x_167; lean_object* x_168; lean_object* x_169; -x_166 = 0; -x_167 = lean_usize_of_nat(x_121); -lean_dec(x_121); -x_168 = lean_box(0); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_68); -x_169 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__8(x_5, x_67, x_68, x_8, x_166, x_167, x_168, x_10, x_11, x_12, x_13, x_14, x_15, x_120); -if (lean_obj_tag(x_169) == 0) -{ -lean_object* x_170; -x_170 = lean_ctor_get(x_169, 1); -lean_inc(x_170); -lean_dec(x_169); -x_123 = x_170; -goto block_164; } else { -uint8_t x_171; -lean_dec(x_94); -lean_dec(x_85); -lean_dec(x_68); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -x_171 = !lean_is_exclusive(x_169); -if (x_171 == 0) +uint8_t x_18; +x_18 = !lean_is_exclusive(x_13); +if (x_18 == 0) { -return x_169; +return x_13; } else { -lean_object* x_172; lean_object* x_173; lean_object* x_174; -x_172 = lean_ctor_get(x_169, 0); -x_173 = lean_ctor_get(x_169, 1); -lean_inc(x_173); -lean_inc(x_172); -lean_dec(x_169); -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_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_13, 0); +x_20 = lean_ctor_get(x_13, 1); +lean_inc(x_20); +lean_inc(x_19); +lean_dec(x_13); +x_21 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_21, 0, x_19); +lean_ctor_set(x_21, 1, x_20); +return x_21; } } } } -block_164: +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: { -lean_object* x_124; size_t x_125; lean_object* x_126; -x_124 = lean_ctor_get(x_12, 1); -lean_inc(x_124); -x_125 = 0; -if (x_96 == 0) +lean_object* x_12; +lean_inc(x_5); +x_12 = l_Lean_mkConstWithLevelParams___at_Lean_Elab_Term_expandDeclId___spec__7(x_1, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_12) == 0) { -lean_object* x_158; -x_158 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; -x_126 = x_158; -goto block_157; -} -else +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_13 = lean_ctor_get(x_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_unsigned_to_nat(1u); +x_16 = l_Lean_Syntax_getArg(x_2, x_15); +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_17 = l_Lean_Elab_Term_addLocalVarInfo(x_16, x_13, x_5, x_6, x_7, x_8, x_9, x_10, x_14); +if (lean_obj_tag(x_17) == 0) { -uint8_t x_159; -x_159 = lean_nat_dec_le(x_94, x_94); -if (x_159 == 0) +lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; lean_object* x_22; +x_18 = lean_ctor_get(x_17, 1); +lean_inc(x_18); +lean_dec(x_17); +x_19 = lean_ctor_get(x_4, 9); +lean_inc(x_19); +lean_dec(x_4); +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +x_21 = 1; +x_22 = l_Lean_Syntax_getPos_x3f(x_20, x_21); +if (lean_obj_tag(x_22) == 0) { -lean_object* x_160; -x_160 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; -x_126 = x_160; -goto block_157; +lean_object* x_23; lean_object* x_24; +lean_dec(x_20); +lean_dec(x_19); +x_23 = lean_box(0); +x_24 = l_Lean_Elab_Command_mkStructureDecl___lambda__1(x_3, x_23, x_5, x_6, x_7, x_8, x_9, x_10, x_18); +return x_24; } else { -size_t x_161; lean_object* x_162; lean_object* x_163; -x_161 = lean_usize_of_nat(x_94); -x_162 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; -x_163 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__7(x_4, x_125, x_161, x_162); -x_126 = x_163; -goto block_157; -} -} -block_157: -{ -size_t x_127; lean_object* x_128; -x_127 = lean_array_size(x_126); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -x_128 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__4(x_127, x_125, x_126, x_10, x_11, x_12, x_13, x_14, x_15, x_123); -if (lean_obj_tag(x_128) == 0) -{ -lean_object* x_129; lean_object* x_130; uint8_t 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 = lean_nat_dec_lt(x_95, x_85); -if (x_131 == 0) +lean_object* x_25; lean_object* x_26; +lean_dec(x_22); +x_25 = lean_ctor_get(x_19, 3); +lean_inc(x_25); +lean_dec(x_19); +lean_inc(x_5); +x_26 = l_Lean_mkConstWithLevelParams___at_Lean_Elab_Term_expandDeclId___spec__7(x_25, x_5, x_6, x_7, x_8, x_9, x_10, x_18); +if (lean_obj_tag(x_26) == 0) { -lean_dec(x_85); -lean_dec(x_68); -if (x_96 == 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_26, 0); +lean_inc(x_27); +x_28 = lean_ctor_get(x_26, 1); +lean_inc(x_28); +lean_dec(x_26); +x_29 = lean_box(0); +x_30 = lean_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_31 = l_Lean_Elab_Term_addTermInfo_x27(x_20, x_27, x_29, x_29, x_30, x_21, x_5, x_6, x_7, x_8, x_9, x_10, x_28); +if (lean_obj_tag(x_31) == 0) { -lean_object* x_132; -lean_dec(x_94); -x_132 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults(x_124, x_129, x_10, x_11, x_12, x_13, x_14, x_15, x_130); -return x_132; +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_31, 0); +lean_inc(x_32); +x_33 = lean_ctor_get(x_31, 1); +lean_inc(x_33); +lean_dec(x_31); +x_34 = l_Lean_Elab_Command_mkStructureDecl___lambda__1(x_3, x_32, x_5, x_6, x_7, x_8, x_9, x_10, x_33); +lean_dec(x_32); +return x_34; } else { -uint8_t x_133; -x_133 = lean_nat_dec_le(x_94, x_94); -if (x_133 == 0) +uint8_t x_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); +x_35 = !lean_is_exclusive(x_31); +if (x_35 == 0) { -lean_object* x_134; -lean_dec(x_94); -x_134 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults(x_124, x_129, x_10, x_11, x_12, x_13, x_14, x_15, x_130); -return x_134; +return x_31; } else { -size_t x_135; lean_object* x_136; lean_object* x_137; -x_135 = lean_usize_of_nat(x_94); -lean_dec(x_94); -x_136 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__5(x_4, x_125, x_135, x_124); -x_137 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults(x_136, x_129, x_10, x_11, x_12, x_13, x_14, x_15, x_130); -return x_137; +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_138; -x_138 = lean_nat_dec_le(x_85, x_85); -if (x_138 == 0) +uint8_t x_39; +lean_dec(x_20); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_39 = !lean_is_exclusive(x_26); +if (x_39 == 0) { -lean_dec(x_85); -lean_dec(x_68); -if (x_96 == 0) +return x_26; +} +else { -lean_object* x_139; -lean_dec(x_94); -x_139 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults(x_124, x_129, x_10, x_11, x_12, x_13, x_14, x_15, x_130); -return x_139; +lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_40 = lean_ctor_get(x_26, 0); +x_41 = lean_ctor_get(x_26, 1); +lean_inc(x_41); +lean_inc(x_40); +lean_dec(x_26); +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_140; -x_140 = lean_nat_dec_le(x_94, x_94); -if (x_140 == 0) +uint8_t x_43; +lean_dec(x_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_43 = !lean_is_exclusive(x_17); +if (x_43 == 0) { -lean_object* x_141; -lean_dec(x_94); -x_141 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults(x_124, x_129, x_10, x_11, x_12, x_13, x_14, x_15, x_130); -return x_141; +return x_17; } else { -size_t x_142; lean_object* x_143; lean_object* x_144; -x_142 = lean_usize_of_nat(x_94); -lean_dec(x_94); -x_143 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__5(x_4, x_125, x_142, x_124); -x_144 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults(x_143, x_129, x_10, x_11, x_12, x_13, x_14, x_15, x_130); -return x_144; +lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_44 = lean_ctor_get(x_17, 0); +x_45 = lean_ctor_get(x_17, 1); +lean_inc(x_45); +lean_inc(x_44); +lean_dec(x_17); +x_46 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_46, 0, x_44); +lean_ctor_set(x_46, 1, x_45); +return x_46; } } } else { -size_t x_145; lean_object* x_146; -x_145 = lean_usize_of_nat(x_85); -lean_dec(x_85); -x_146 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__6(x_68, x_125, x_145, x_124); -lean_dec(x_68); -if (x_96 == 0) +uint8_t x_47; +lean_dec(x_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_47 = !lean_is_exclusive(x_12); +if (x_47 == 0) { -lean_object* x_147; -lean_dec(x_94); -x_147 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults(x_146, x_129, x_10, x_11, x_12, x_13, x_14, x_15, x_130); -return x_147; +return x_12; } else { -uint8_t x_148; -x_148 = lean_nat_dec_le(x_94, x_94); -if (x_148 == 0) -{ -lean_object* x_149; -lean_dec(x_94); -x_149 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults(x_146, x_129, x_10, x_11, x_12, x_13, x_14, x_15, x_130); -return x_149; +lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_48 = lean_ctor_get(x_12, 0); +x_49 = lean_ctor_get(x_12, 1); +lean_inc(x_49); +lean_inc(x_48); +lean_dec(x_12); +x_50 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_50, 0, x_48); +lean_ctor_set(x_50, 1, x_49); +return x_50; } -else -{ -size_t x_150; lean_object* x_151; lean_object* x_152; -x_150 = lean_usize_of_nat(x_94); -lean_dec(x_94); -x_151 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__5(x_4, x_125, x_150, x_146); -x_152 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults(x_151, x_129, x_10, x_11, x_12, x_13, x_14, x_15, x_130); -return x_152; } } } +static lean_object* _init_l_Lean_Elab_Command_mkStructureDecl___lambda__3___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_withSaveInfoContext___at___private_Lean_Elab_PreDefinition_Basic_0__Lean_Elab_addNonRecAux___spec__1___lambda__1___boxed), 7, 0); +return x_1; } } -else +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18) { +_start: { -uint8_t x_153; -lean_dec(x_124); -lean_dec(x_94); -lean_dec(x_85); -lean_dec(x_68); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -x_153 = !lean_is_exclusive(x_128); -if (x_153 == 0) +lean_object* x_19; +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_12); +lean_inc(x_1); +x_19 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections(x_1, x_2, x_12, x_13, x_14, x_15, x_16, x_17, x_18); +if (lean_obj_tag(x_19) == 0) +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_19, 1); +lean_inc(x_20); +lean_dec(x_19); +x_21 = lean_ctor_get(x_3, 4); +lean_inc(x_21); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_21); +x_22 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure(x_21, x_2, x_12, x_13, x_14, x_15, x_16, x_17, x_20); +if (lean_obj_tag(x_22) == 0) { -return x_128; +lean_object* x_23; lean_object* x_24; +x_23 = lean_ctor_get(x_22, 1); +lean_inc(x_23); +lean_dec(x_22); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_21); +x_24 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions(x_21, x_12, x_13, x_14, x_15, x_16, x_17, x_23); +if (lean_obj_tag(x_24) == 0) +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; lean_object* x_30; lean_object* x_31; +x_25 = lean_ctor_get(x_24, 1); +lean_inc(x_25); +lean_dec(x_24); +x_26 = lean_array_get_size(x_2); +lean_inc(x_4); +x_27 = lean_array_mk(x_4); +x_28 = lean_unsigned_to_nat(0u); +x_29 = lean_nat_dec_lt(x_28, x_26); +if (x_29 == 0) +{ +x_30 = x_27; +x_31 = x_25; +goto block_113; } else { -lean_object* x_154; lean_object* x_155; lean_object* x_156; -x_154 = lean_ctor_get(x_128, 0); -x_155 = lean_ctor_get(x_128, 1); -lean_inc(x_155); -lean_inc(x_154); -lean_dec(x_128); -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; -} -} -} +uint8_t x_114; +x_114 = lean_nat_dec_le(x_26, x_26); +if (x_114 == 0) +{ +x_30 = x_27; +x_31 = x_25; +goto block_113; } +else +{ +size_t x_115; size_t x_116; lean_object* x_117; +x_115 = 0; +x_116 = lean_usize_of_nat(x_26); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +x_117 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_mkStructureDecl___spec__6(x_2, x_115, x_116, x_27, x_12, x_13, x_14, x_15, x_16, x_17, x_25); +if (lean_obj_tag(x_117) == 0) +{ +lean_object* x_118; lean_object* x_119; +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_30 = x_118; +x_31 = x_119; +goto block_113; } else { -uint8_t x_175; -lean_dec(x_94); -lean_dec(x_85); -lean_dec(x_68); -lean_dec(x_67); +uint8_t x_120; +lean_dec(x_26); +lean_dec(x_21); +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_7); +lean_dec(x_6); lean_dec(x_5); -x_175 = !lean_is_exclusive(x_119); -if (x_175 == 0) +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_120 = !lean_is_exclusive(x_117); +if (x_120 == 0) { -return x_119; +return x_117; } else { -lean_object* x_176; lean_object* x_177; lean_object* x_178; -x_176 = lean_ctor_get(x_119, 0); -x_177 = lean_ctor_get(x_119, 1); -lean_inc(x_177); -lean_inc(x_176); -lean_dec(x_119); -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; +lean_object* x_121; lean_object* x_122; lean_object* x_123; +x_121 = lean_ctor_get(x_117, 0); +x_122 = lean_ctor_get(x_117, 1); +lean_inc(x_122); +lean_inc(x_121); +lean_dec(x_117); +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 +} +block_113: { -uint8_t x_179; -lean_dec(x_107); -lean_dec(x_94); -lean_dec(x_85); -lean_dec(x_68); -lean_dec(x_67); -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_5); -x_179 = !lean_is_exclusive(x_115); -if (x_179 == 0) +lean_object* x_32; lean_object* x_33; lean_object* x_34; +lean_inc(x_3); +lean_inc(x_21); +x_32 = lean_alloc_closure((void*)(l_Lean_Elab_Command_mkStructureDecl___lambda__2___boxed), 11, 4); +lean_closure_set(x_32, 0, x_21); +lean_closure_set(x_32, 1, x_5); +lean_closure_set(x_32, 2, x_6); +lean_closure_set(x_32, 3, x_3); +x_33 = l_Lean_Elab_Command_mkStructureDecl___lambda__3___closed__1; +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_34 = l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at___private_Lean_Elab_PreDefinition_Basic_0__Lean_Elab_addNonRecAux___spec__2(x_32, x_33, x_12, x_13, x_14, x_15, x_16, x_17, x_31); +if (lean_obj_tag(x_34) == 0) +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; lean_object* x_49; uint8_t x_50; lean_object* x_51; lean_object* x_52; uint8_t x_53; lean_object* x_54; +x_35 = lean_ctor_get(x_34, 1); +lean_inc(x_35); +lean_dec(x_34); +x_36 = lean_ctor_get(x_7, 2); +lean_inc(x_36); +lean_dec(x_7); +x_37 = lean_ctor_get(x_16, 0); +lean_inc(x_37); +x_38 = lean_ctor_get(x_16, 1); +lean_inc(x_38); +x_39 = lean_ctor_get(x_16, 2); +lean_inc(x_39); +x_40 = lean_ctor_get(x_16, 3); +lean_inc(x_40); +x_41 = lean_ctor_get(x_16, 4); +lean_inc(x_41); +x_42 = lean_ctor_get(x_16, 5); +lean_inc(x_42); +x_43 = lean_ctor_get(x_16, 6); +lean_inc(x_43); +x_44 = lean_ctor_get(x_16, 7); +lean_inc(x_44); +x_45 = lean_ctor_get(x_16, 8); +lean_inc(x_45); +x_46 = lean_ctor_get(x_16, 9); +lean_inc(x_46); +x_47 = lean_ctor_get(x_16, 10); +lean_inc(x_47); +x_48 = lean_ctor_get_uint8(x_16, sizeof(void*)*12); +x_49 = lean_ctor_get(x_16, 11); +lean_inc(x_49); +x_50 = lean_ctor_get_uint8(x_16, sizeof(void*)*12 + 1); +x_51 = l_Lean_replaceRef(x_8, x_42); +lean_dec(x_42); +x_52 = lean_alloc_ctor(0, 12, 2); +lean_ctor_set(x_52, 0, x_37); +lean_ctor_set(x_52, 1, x_38); +lean_ctor_set(x_52, 2, x_39); +lean_ctor_set(x_52, 3, x_40); +lean_ctor_set(x_52, 4, x_41); +lean_ctor_set(x_52, 5, x_51); +lean_ctor_set(x_52, 6, x_43); +lean_ctor_set(x_52, 7, x_44); +lean_ctor_set(x_52, 8, x_45); +lean_ctor_set(x_52, 9, x_46); +lean_ctor_set(x_52, 10, x_47); +lean_ctor_set(x_52, 11, x_49); +lean_ctor_set_uint8(x_52, sizeof(void*)*12, x_48); +lean_ctor_set_uint8(x_52, sizeof(void*)*12 + 1, x_50); +x_53 = 0; +lean_inc(x_17); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +x_54 = l_Lean_Elab_Term_applyAttributesAt(x_21, x_36, x_53, x_12, x_13, x_14, x_15, x_52, x_17, x_35); +if (lean_obj_tag(x_54) == 0) +{ +lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; +x_55 = lean_ctor_get(x_54, 1); +lean_inc(x_55); +lean_dec(x_54); +x_56 = lean_array_to_list(x_30); +x_57 = l_List_mapTR_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__1(x_56, x_4); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +x_58 = l_List_forM___at_Lean_Elab_Command_mkStructureDecl___spec__2(x_57, x_12, x_13, x_14, x_15, x_16, x_17, x_55); +if (lean_obj_tag(x_58) == 0) +{ +lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; lean_object* x_63; +x_59 = lean_ctor_get(x_58, 1); +lean_inc(x_59); +lean_dec(x_58); +x_60 = lean_ctor_get(x_1, 6); +lean_inc(x_60); +lean_dec(x_1); +x_61 = lean_array_get_size(x_60); +x_62 = lean_nat_dec_lt(x_28, x_61); +if (x_62 == 0) { -return x_115; +lean_dec(x_61); +lean_dec(x_60); +lean_dec(x_11); +lean_dec(x_3); +x_63 = x_59; +goto block_90; } else { -lean_object* x_180; lean_object* x_181; lean_object* x_182; -x_180 = lean_ctor_get(x_115, 0); -x_181 = lean_ctor_get(x_115, 1); -lean_inc(x_181); -lean_inc(x_180); -lean_dec(x_115); -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; -} +uint8_t x_91; +x_91 = lean_nat_dec_le(x_61, x_61); +if (x_91 == 0) +{ +lean_dec(x_61); +lean_dec(x_60); +lean_dec(x_11); +lean_dec(x_3); +x_63 = x_59; +goto block_90; } +else +{ +size_t x_92; size_t x_93; lean_object* x_94; lean_object* x_95; +x_92 = 0; +x_93 = lean_usize_of_nat(x_61); +lean_dec(x_61); +x_94 = lean_box(0); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_10); +x_95 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_mkStructureDecl___spec__5(x_3, x_11, x_10, x_60, x_92, x_93, x_94, x_12, x_13, x_14, x_15, x_16, x_17, x_59); +lean_dec(x_60); +if (lean_obj_tag(x_95) == 0) +{ +lean_object* x_96; +x_96 = lean_ctor_get(x_95, 1); +lean_inc(x_96); +lean_dec(x_95); +x_63 = x_96; +goto block_90; } else { -uint8_t x_183; -lean_dec(x_107); -lean_dec(x_94); -lean_dec(x_87); -lean_dec(x_85); -lean_dec(x_82); -lean_dec(x_68); -lean_dec(x_67); +uint8_t x_97; +lean_dec(x_26); +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_5); -x_183 = !lean_is_exclusive(x_111); -if (x_183 == 0) +lean_dec(x_2); +x_97 = !lean_is_exclusive(x_95); +if (x_97 == 0) { -return x_111; +return x_95; } else { -lean_object* x_184; lean_object* x_185; lean_object* x_186; -x_184 = lean_ctor_get(x_111, 0); -x_185 = lean_ctor_get(x_111, 1); -lean_inc(x_185); -lean_inc(x_184); -lean_dec(x_111); -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_98; lean_object* x_99; lean_object* x_100; +x_98 = lean_ctor_get(x_95, 0); +x_99 = lean_ctor_get(x_95, 1); +lean_inc(x_99); +lean_inc(x_98); +lean_dec(x_95); +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 +block_90: +{ +lean_object* x_64; uint8_t x_65; +x_64 = lean_ctor_get(x_14, 1); +lean_inc(x_64); +x_65 = lean_nat_dec_lt(x_28, x_9); +if (x_65 == 0) { -uint8_t x_201; -lean_dec(x_94); -lean_dec(x_87); -lean_dec(x_85); -lean_dec(x_82); -lean_dec(x_68); -lean_dec(x_67); -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_7); -lean_dec(x_6); -lean_dec(x_5); -x_201 = !lean_is_exclusive(x_105); -if (x_201 == 0) +if (x_29 == 0) { -return x_105; +lean_object* x_66; +lean_dec(x_26); +x_66 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults(x_64, x_2, x_12, x_13, x_14, x_15, x_16, x_17, x_63); +return x_66; } else { -lean_object* x_202; lean_object* x_203; lean_object* x_204; -x_202 = lean_ctor_get(x_105, 0); -x_203 = lean_ctor_get(x_105, 1); -lean_inc(x_203); -lean_inc(x_202); -lean_dec(x_105); -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; +uint8_t x_67; +x_67 = lean_nat_dec_le(x_26, x_26); +if (x_67 == 0) +{ +lean_object* x_68; +lean_dec(x_26); +x_68 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults(x_64, x_2, x_12, x_13, x_14, x_15, x_16, x_17, x_63); +return x_68; +} +else +{ +size_t x_69; size_t x_70; lean_object* x_71; lean_object* x_72; +x_69 = 0; +x_70 = lean_usize_of_nat(x_26); +lean_dec(x_26); +x_71 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_mkStructureDecl___spec__3(x_2, x_69, x_70, x_64); +x_72 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults(x_71, x_2, x_12, x_13, x_14, x_15, x_16, x_17, x_63); +return x_72; } } } else { -uint8_t x_205; -lean_dec(x_94); -lean_dec(x_87); -lean_dec(x_85); -lean_dec(x_82); -lean_dec(x_68); -lean_dec(x_67); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); +uint8_t x_73; +x_73 = lean_nat_dec_le(x_9, x_9); +if (x_73 == 0) +{ lean_dec(x_10); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -x_205 = !lean_is_exclusive(x_103); -if (x_205 == 0) +if (x_29 == 0) { -return x_103; +lean_object* x_74; +lean_dec(x_26); +x_74 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults(x_64, x_2, x_12, x_13, x_14, x_15, x_16, x_17, x_63); +return x_74; } else { -lean_object* x_206; lean_object* x_207; lean_object* x_208; -x_206 = lean_ctor_get(x_103, 0); -x_207 = lean_ctor_get(x_103, 1); -lean_inc(x_207); -lean_inc(x_206); -lean_dec(x_103); -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; +uint8_t x_75; +x_75 = lean_nat_dec_le(x_26, x_26); +if (x_75 == 0) +{ +lean_object* x_76; +lean_dec(x_26); +x_76 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults(x_64, x_2, x_12, x_13, x_14, x_15, x_16, x_17, x_63); +return x_76; +} +else +{ +size_t x_77; size_t x_78; lean_object* x_79; lean_object* x_80; +x_77 = 0; +x_78 = lean_usize_of_nat(x_26); +lean_dec(x_26); +x_79 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_mkStructureDecl___spec__3(x_2, x_77, x_78, x_64); +x_80 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults(x_79, x_2, x_12, x_13, x_14, x_15, x_16, x_17, x_63); +return x_80; } } } else { -uint8_t x_209; -lean_dec(x_94); -lean_dec(x_87); -lean_dec(x_85); -lean_dec(x_82); -lean_dec(x_68); -lean_dec(x_67); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); +size_t x_81; size_t x_82; lean_object* x_83; +x_81 = 0; +x_82 = lean_usize_of_nat(x_9); +x_83 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_mkStructureDecl___spec__4(x_10, x_81, x_82, x_64); lean_dec(x_10); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -x_209 = !lean_is_exclusive(x_101); -if (x_209 == 0) +if (x_29 == 0) { -return x_101; +lean_object* x_84; +lean_dec(x_26); +x_84 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults(x_83, x_2, x_12, x_13, x_14, x_15, x_16, x_17, x_63); +return x_84; } else { -lean_object* x_210; lean_object* x_211; lean_object* x_212; -x_210 = lean_ctor_get(x_101, 0); -x_211 = lean_ctor_get(x_101, 1); -lean_inc(x_211); -lean_inc(x_210); -lean_dec(x_101); -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; +uint8_t x_85; +x_85 = lean_nat_dec_le(x_26, x_26); +if (x_85 == 0) +{ +lean_object* x_86; +lean_dec(x_26); +x_86 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults(x_83, x_2, x_12, x_13, x_14, x_15, x_16, x_17, x_63); +return x_86; +} +else +{ +size_t x_87; lean_object* x_88; lean_object* x_89; +x_87 = lean_usize_of_nat(x_26); +lean_dec(x_26); +x_88 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_mkStructureDecl___spec__3(x_2, x_81, x_87, x_83); +x_89 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults(x_88, x_2, x_12, x_13, x_14, x_15, x_16, x_17, x_63); +return x_89; +} +} } } } } else { -uint8_t x_221; -lean_dec(x_87); -lean_dec(x_85); -lean_dec(x_82); -lean_dec(x_68); -lean_dec(x_67); +uint8_t x_101; +lean_dec(x_26); +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_7); -lean_dec(x_6); -lean_dec(x_5); -x_221 = !lean_is_exclusive(x_92); -if (x_221 == 0) +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_101 = !lean_is_exclusive(x_58); +if (x_101 == 0) { -return x_92; +return x_58; } else { -lean_object* x_222; lean_object* x_223; lean_object* x_224; -x_222 = lean_ctor_get(x_92, 0); -x_223 = lean_ctor_get(x_92, 1); -lean_inc(x_223); -lean_inc(x_222); -lean_dec(x_92); -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_102; lean_object* x_103; lean_object* x_104; +x_102 = lean_ctor_get(x_58, 0); +x_103 = lean_ctor_get(x_58, 1); +lean_inc(x_103); +lean_inc(x_102); +lean_dec(x_58); +x_104 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_104, 0, x_102); +lean_ctor_set(x_104, 1, x_103); +return x_104; } } } else { -uint8_t x_225; -lean_dec(x_89); -lean_dec(x_87); -lean_dec(x_85); -lean_dec(x_82); -lean_dec(x_68); -lean_dec(x_67); +uint8_t x_105; +lean_dec(x_30); +lean_dec(x_26); +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_7); -lean_dec(x_6); -lean_dec(x_5); -x_225 = !lean_is_exclusive(x_90); -if (x_225 == 0) +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_105 = !lean_is_exclusive(x_54); +if (x_105 == 0) { -return x_90; +return x_54; } else { -lean_object* x_226; lean_object* x_227; lean_object* x_228; -x_226 = lean_ctor_get(x_90, 0); -x_227 = lean_ctor_get(x_90, 1); -lean_inc(x_227); -lean_inc(x_226); -lean_dec(x_90); -x_228 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_228, 0, x_226); -lean_ctor_set(x_228, 1, x_227); -return x_228; -} +lean_object* x_106; lean_object* x_107; lean_object* x_108; +x_106 = lean_ctor_get(x_54, 0); +x_107 = lean_ctor_get(x_54, 1); +lean_inc(x_107); +lean_inc(x_106); +lean_dec(x_54); +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 -{ -lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; uint8_t x_238; lean_object* x_239; lean_object* x_240; -x_229 = lean_ctor_get(x_78, 0); -x_230 = lean_ctor_get(x_78, 1); -lean_inc(x_230); -lean_inc(x_229); -lean_dec(x_78); -x_231 = lean_ctor_get(x_5, 4); -lean_inc(x_231); -x_232 = lean_box(0); -x_233 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_233, 0, x_70); -lean_ctor_set(x_233, 1, x_232); -lean_inc(x_231); -x_234 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_234, 0, x_231); -lean_ctor_set(x_234, 1, x_229); -lean_ctor_set(x_234, 2, x_233); -x_235 = lean_array_get_size(x_68); -x_236 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_236, 0, x_234); -lean_ctor_set(x_236, 1, x_232); -x_237 = lean_ctor_get(x_5, 1); -lean_inc(x_237); -x_238 = lean_ctor_get_uint8(x_237, sizeof(void*)*2 + 3); -lean_inc(x_235); -lean_inc(x_67); -x_239 = lean_alloc_ctor(6, 3, 1); -lean_ctor_set(x_239, 0, x_67); -lean_ctor_set(x_239, 1, x_235); -lean_ctor_set(x_239, 2, x_236); -lean_ctor_set_uint8(x_239, sizeof(void*)*3, x_238); -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_239); -x_240 = l_Lean_Elab_Term_ensureNoUnassignedMVars(x_239, x_10, x_11, x_12, x_13, x_14, x_15, x_230); -if (lean_obj_tag(x_240) == 0) -{ -lean_object* x_241; lean_object* x_242; -x_241 = lean_ctor_get(x_240, 1); -lean_inc(x_241); -lean_dec(x_240); -lean_inc(x_15); -lean_inc(x_14); -x_242 = l_Lean_addDecl(x_239, x_14, x_15, x_241); -if (lean_obj_tag(x_242) == 0) -{ -lean_object* x_243; lean_object* x_244; lean_object* x_245; uint8_t x_246; uint8_t x_247; lean_object* x_248; -x_243 = lean_ctor_get(x_242, 1); -lean_inc(x_243); -lean_dec(x_242); -x_244 = lean_array_get_size(x_4); -x_245 = lean_unsigned_to_nat(0u); -x_246 = lean_nat_dec_lt(x_245, x_244); -x_247 = lean_ctor_get_uint8(x_5, sizeof(void*)*11); -if (x_246 == 0) -{ -lean_object* x_364; -x_364 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; -x_248 = x_364; -goto block_363; } else { -uint8_t x_365; -x_365 = lean_nat_dec_le(x_244, x_244); -if (x_365 == 0) +uint8_t x_109; +lean_dec(x_30); +lean_dec(x_26); +lean_dec(x_21); +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_7); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_109 = !lean_is_exclusive(x_34); +if (x_109 == 0) { -lean_object* x_366; -x_366 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; -x_248 = x_366; -goto block_363; +return x_34; } else { -size_t x_367; size_t x_368; lean_object* x_369; lean_object* x_370; -x_367 = 0; -x_368 = lean_usize_of_nat(x_244); -x_369 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; -x_370 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__10(x_4, x_367, x_368, x_369); -x_248 = x_370; -goto block_363; -} +lean_object* x_110; lean_object* x_111; lean_object* x_112; +x_110 = lean_ctor_get(x_34, 0); +x_111 = lean_ctor_get(x_34, 1); +lean_inc(x_111); +lean_inc(x_110); +lean_dec(x_34); +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; } -block_363: -{ -lean_object* x_249; lean_object* x_250; lean_object* x_251; -x_249 = lean_array_to_list(x_248); -x_250 = l_List_mapTR_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__1(x_249, x_232); -lean_inc(x_14); -lean_inc(x_10); -lean_inc(x_231); -x_251 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections(x_231, x_250, x_247, x_10, x_11, x_12, x_13, x_14, x_15, x_243); -if (lean_obj_tag(x_251) == 0) -{ -lean_object* x_252; lean_object* x_253; -x_252 = lean_ctor_get(x_251, 1); -lean_inc(x_252); -lean_dec(x_251); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_231); -x_253 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure(x_231, x_4, x_10, x_11, x_12, x_13, x_14, x_15, x_252); -if (lean_obj_tag(x_253) == 0) -{ -lean_object* x_254; lean_object* x_255; -x_254 = lean_ctor_get(x_253, 1); -lean_inc(x_254); -lean_dec(x_253); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_231); -x_255 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions(x_231, x_10, x_11, x_12, x_13, x_14, x_15, x_254); -if (lean_obj_tag(x_255) == 0) -{ -lean_object* x_256; lean_object* x_257; lean_object* x_258; -x_256 = lean_ctor_get(x_255, 1); -lean_inc(x_256); -lean_dec(x_255); -if (x_246 == 0) -{ -lean_object* x_338; -x_338 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; -x_257 = x_338; -x_258 = x_256; -goto block_337; } -else -{ -uint8_t x_339; -x_339 = lean_nat_dec_le(x_244, x_244); -if (x_339 == 0) -{ -lean_object* x_340; -x_340 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; -x_257 = x_340; -x_258 = x_256; -goto block_337; } -else -{ -size_t x_341; size_t x_342; lean_object* x_343; lean_object* x_344; -x_341 = 0; -x_342 = lean_usize_of_nat(x_244); -x_343 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; -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_344 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__9(x_4, x_341, x_342, x_343, x_10, x_11, x_12, x_13, x_14, x_15, x_256); -if (lean_obj_tag(x_344) == 0) -{ -lean_object* x_345; lean_object* x_346; -x_345 = lean_ctor_get(x_344, 0); -lean_inc(x_345); -x_346 = lean_ctor_get(x_344, 1); -lean_inc(x_346); -lean_dec(x_344); -x_257 = x_345; -x_258 = x_346; -goto block_337; } else { -lean_object* x_347; lean_object* x_348; lean_object* x_349; lean_object* x_350; -lean_dec(x_244); -lean_dec(x_237); -lean_dec(x_235); -lean_dec(x_231); -lean_dec(x_68); -lean_dec(x_67); +uint8_t x_124; +lean_dec(x_21); +lean_dec(x_17); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -31961,790 +31011,986 @@ lean_dec(x_10); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -x_347 = lean_ctor_get(x_344, 0); -lean_inc(x_347); -x_348 = lean_ctor_get(x_344, 1); -lean_inc(x_348); -if (lean_is_exclusive(x_344)) { - lean_ctor_release(x_344, 0); - lean_ctor_release(x_344, 1); - x_349 = x_344; -} else { - lean_dec_ref(x_344); - x_349 = lean_box(0); -} -if (lean_is_scalar(x_349)) { - x_350 = lean_alloc_ctor(1, 2, 0); -} else { - x_350 = x_349; -} -lean_ctor_set(x_350, 0, x_347); -lean_ctor_set(x_350, 1, x_348); -return x_350; -} -} -} -block_337: -{ -lean_object* x_259; lean_object* x_260; lean_object* x_261; -lean_inc(x_5); -lean_inc(x_231); -x_259 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__2___boxed), 11, 4); -lean_closure_set(x_259, 0, x_231); -lean_closure_set(x_259, 1, x_6); -lean_closure_set(x_259, 2, x_7); -lean_closure_set(x_259, 3, x_5); -x_260 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__3___closed__1; -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_261 = l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at___private_Lean_Elab_PreDefinition_Basic_0__Lean_Elab_addNonRecAux___spec__2(x_259, x_260, x_10, x_11, x_12, x_13, x_14, x_15, x_258); -if (lean_obj_tag(x_261) == 0) -{ -lean_object* x_262; lean_object* x_263; uint8_t x_264; lean_object* x_265; -x_262 = lean_ctor_get(x_261, 1); -lean_inc(x_262); -lean_dec(x_261); -x_263 = lean_ctor_get(x_237, 1); -lean_inc(x_263); -lean_dec(x_237); -x_264 = 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_265 = l_Lean_Elab_Term_applyAttributesAt(x_231, x_263, x_264, x_10, x_11, x_12, x_13, x_14, x_15, x_262); -if (lean_obj_tag(x_265) == 0) -{ -lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; -x_266 = lean_ctor_get(x_265, 1); -lean_inc(x_266); -lean_dec(x_265); -x_267 = lean_array_to_list(x_257); -x_268 = l_List_mapTR_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__1(x_267, x_232); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -x_269 = l_List_forM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__3(x_268, x_10, x_11, x_12, x_13, x_14, x_15, x_266); -if (lean_obj_tag(x_269) == 0) -{ -lean_object* x_270; lean_object* x_271; uint8_t x_272; lean_object* x_273; -x_270 = lean_ctor_get(x_269, 1); -lean_inc(x_270); -lean_dec(x_269); -x_271 = lean_array_get_size(x_8); -x_272 = lean_nat_dec_lt(x_245, x_271); -if (x_272 == 0) +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_124 = !lean_is_exclusive(x_24); +if (x_124 == 0) { -lean_dec(x_271); -lean_dec(x_67); -lean_dec(x_5); -x_273 = x_270; -goto block_314; +return x_24; } else { -uint8_t x_315; -x_315 = lean_nat_dec_le(x_271, x_271); -if (x_315 == 0) -{ -lean_dec(x_271); -lean_dec(x_67); -lean_dec(x_5); -x_273 = x_270; -goto block_314; +lean_object* x_125; lean_object* x_126; lean_object* x_127; +x_125 = lean_ctor_get(x_24, 0); +x_126 = lean_ctor_get(x_24, 1); +lean_inc(x_126); +lean_inc(x_125); +lean_dec(x_24); +x_127 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_127, 0, x_125); +lean_ctor_set(x_127, 1, x_126); +return x_127; +} } -else -{ -size_t x_316; size_t x_317; lean_object* x_318; lean_object* x_319; -x_316 = 0; -x_317 = lean_usize_of_nat(x_271); -lean_dec(x_271); -x_318 = lean_box(0); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_68); -x_319 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__8(x_5, x_67, x_68, x_8, x_316, x_317, x_318, x_10, x_11, x_12, x_13, x_14, x_15, x_270); -if (lean_obj_tag(x_319) == 0) -{ -lean_object* x_320; -x_320 = lean_ctor_get(x_319, 1); -lean_inc(x_320); -lean_dec(x_319); -x_273 = x_320; -goto block_314; } else { -lean_object* x_321; lean_object* x_322; lean_object* x_323; lean_object* x_324; -lean_dec(x_244); -lean_dec(x_235); -lean_dec(x_68); +uint8_t x_128; +lean_dec(x_21); +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); -x_321 = lean_ctor_get(x_319, 0); -lean_inc(x_321); -x_322 = lean_ctor_get(x_319, 1); -lean_inc(x_322); -if (lean_is_exclusive(x_319)) { - lean_ctor_release(x_319, 0); - lean_ctor_release(x_319, 1); - x_323 = x_319; -} else { - lean_dec_ref(x_319); - x_323 = lean_box(0); -} -if (lean_is_scalar(x_323)) { - x_324 = lean_alloc_ctor(1, 2, 0); -} else { - x_324 = x_323; -} -lean_ctor_set(x_324, 0, x_321); -lean_ctor_set(x_324, 1, x_322); -return x_324; +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_128 = !lean_is_exclusive(x_22); +if (x_128 == 0) +{ +return x_22; } +else +{ +lean_object* x_129; lean_object* x_130; lean_object* x_131; +x_129 = lean_ctor_get(x_22, 0); +x_130 = lean_ctor_get(x_22, 1); +lean_inc(x_130); +lean_inc(x_129); +lean_dec(x_22); +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; } } -block_314: -{ -lean_object* x_274; size_t x_275; lean_object* x_276; -x_274 = lean_ctor_get(x_12, 1); -lean_inc(x_274); -x_275 = 0; -if (x_246 == 0) -{ -lean_object* x_308; -x_308 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; -x_276 = x_308; -goto block_307; } else { -uint8_t x_309; -x_309 = lean_nat_dec_le(x_244, x_244); -if (x_309 == 0) +uint8_t x_132; +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_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_132 = !lean_is_exclusive(x_19); +if (x_132 == 0) { -lean_object* x_310; -x_310 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; -x_276 = x_310; -goto block_307; +return x_19; } else { -size_t x_311; lean_object* x_312; lean_object* x_313; -x_311 = lean_usize_of_nat(x_244); -x_312 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; -x_313 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__7(x_4, x_275, x_311, x_312); -x_276 = x_313; -goto block_307; +lean_object* x_133; lean_object* x_134; lean_object* x_135; +x_133 = lean_ctor_get(x_19, 0); +x_134 = lean_ctor_get(x_19, 1); +lean_inc(x_134); +lean_inc(x_133); +lean_dec(x_19); +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; +} } } -block_307: +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, uint8_t x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19, lean_object* x_20, lean_object* x_21) { +_start: { -size_t x_277; lean_object* x_278; -x_277 = lean_array_size(x_276); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -x_278 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__4(x_277, x_275, x_276, x_10, x_11, x_12, x_13, x_14, x_15, x_273); -if (lean_obj_tag(x_278) == 0) -{ -lean_object* x_279; lean_object* x_280; uint8_t x_281; -x_279 = lean_ctor_get(x_278, 0); -lean_inc(x_279); -x_280 = lean_ctor_get(x_278, 1); -lean_inc(x_280); -lean_dec(x_278); -x_281 = lean_nat_dec_lt(x_245, x_235); -if (x_281 == 0) -{ -lean_dec(x_235); -lean_dec(x_68); -if (x_246 == 0) +lean_object* x_22; +lean_inc(x_20); +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_1); +x_22 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectLevelParamsInStructure(x_1, x_2, x_3, x_4, x_15, x_16, x_17, x_18, x_19, x_20, x_21); +if (lean_obj_tag(x_22) == 0) { -lean_object* x_282; -lean_dec(x_244); -x_282 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults(x_274, x_279, x_10, x_11, x_12, x_13, x_14, x_15, x_280); -return x_282; -} -else +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +lean_dec(x_22); +x_25 = lean_ctor_get(x_5, 3); +lean_inc(x_25); +x_26 = l_Lean_Elab_sortDeclLevelParams(x_6, x_25, x_23); +if (lean_obj_tag(x_26) == 0) { -uint8_t x_283; -x_283 = lean_nat_dec_le(x_244, x_244); -if (x_283 == 0) +uint8_t x_27; +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_27 = !lean_is_exclusive(x_26); +if (x_27 == 0) { -lean_object* x_284; -lean_dec(x_244); -x_284 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults(x_274, x_279, x_10, x_11, x_12, x_13, x_14, x_15, x_280); -return x_284; +lean_object* x_28; lean_object* x_29; +lean_ctor_set_tag(x_26, 3); +x_28 = l_Lean_MessageData_ofFormat(x_26); +x_29 = l_Lean_throwErrorAt___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__12(x_7, x_28, x_15, x_16, x_17, x_18, x_19, x_20, x_24); +lean_dec(x_20); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_7); +return x_29; } else { -size_t x_285; lean_object* x_286; lean_object* x_287; -x_285 = lean_usize_of_nat(x_244); -lean_dec(x_244); -x_286 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__5(x_4, x_275, x_285, x_274); -x_287 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults(x_286, x_279, x_10, x_11, x_12, x_13, x_14, x_15, x_280); -return x_287; -} +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_30 = lean_ctor_get(x_26, 0); +lean_inc(x_30); +lean_dec(x_26); +x_31 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_31, 0, x_30); +x_32 = l_Lean_MessageData_ofFormat(x_31); +x_33 = l_Lean_throwErrorAt___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__12(x_7, x_32, x_15, x_16, x_17, x_18, x_19, x_20, x_24); +lean_dec(x_20); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_7); +return x_33; } } else { -uint8_t x_288; -x_288 = lean_nat_dec_le(x_235, x_235); -if (x_288 == 0) +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_26, 0); +lean_inc(x_34); +lean_dec(x_26); +lean_inc(x_2); +x_35 = l_Array_append___rarg(x_2, x_3); +lean_inc(x_20); +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_35); +lean_inc(x_34); +lean_inc(x_8); +x_36 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCtor(x_8, x_34, x_35, x_4, x_15, x_16, x_17, x_18, x_19, x_20, x_24); +if (lean_obj_tag(x_36) == 0) +{ +lean_object* x_37; lean_object* x_38; uint8_t x_39; uint8_t x_40; uint8_t x_41; lean_object* x_42; +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 = 0; +x_40 = 1; +x_41 = 1; +lean_inc(x_35); +x_42 = l_Lean_Meta_mkForallFVars(x_35, x_1, x_39, x_40, x_41, x_17, x_18, x_19, x_20, x_38); +if (lean_obj_tag(x_42) == 0) { -lean_dec(x_235); -lean_dec(x_68); -if (x_246 == 0) +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); +x_45 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_43, x_15, x_16, x_17, x_18, x_19, x_20, x_44); +x_46 = !lean_is_exclusive(x_45); +if (x_46 == 0) { -lean_object* x_289; -lean_dec(x_244); -x_289 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults(x_274, x_279, x_10, x_11, x_12, x_13, x_14, x_15, x_280); -return x_289; -} -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_45, 0); +x_48 = lean_ctor_get(x_45, 1); +x_49 = lean_array_get_size(x_2); +lean_dec(x_2); +x_50 = lean_array_get_size(x_35); +lean_inc(x_20); +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_50); +lean_inc(x_34); +lean_inc(x_9); +lean_inc(x_8); +x_51 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkInductiveType(x_8, x_9, x_34, x_49, x_50, x_47, x_37, x_15, x_16, x_17, x_18, x_19, x_20, x_48); +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; +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_box(0); +lean_ctor_set_tag(x_45, 1); +lean_ctor_set(x_45, 1, x_54); +lean_ctor_set(x_45, 0, x_52); +lean_inc(x_50); +lean_inc(x_34); +x_55 = lean_alloc_ctor(6, 3, 1); +lean_ctor_set(x_55, 0, x_34); +lean_ctor_set(x_55, 1, x_50); +lean_ctor_set(x_55, 2, x_45); +lean_ctor_set_uint8(x_55, sizeof(void*)*3, x_10); +lean_inc(x_20); +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_55); +x_56 = l_Lean_Elab_Term_ensureNoUnassignedMVars(x_55, x_15, x_16, x_17, x_18, x_19, x_20, x_53); +if (lean_obj_tag(x_56) == 0) { -uint8_t x_290; -x_290 = lean_nat_dec_le(x_244, x_244); -if (x_290 == 0) +lean_object* x_57; lean_object* x_58; +x_57 = lean_ctor_get(x_56, 1); +lean_inc(x_57); +lean_dec(x_56); +lean_inc(x_20); +lean_inc(x_19); +x_58 = l_Lean_addDecl(x_55, x_19, x_20, x_57); +if (lean_obj_tag(x_58) == 0) { -lean_object* x_291; -lean_dec(x_244); -x_291 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults(x_274, x_279, x_10, x_11, x_12, x_13, x_14, x_15, x_280); -return x_291; -} -else +lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_59 = lean_ctor_get(x_58, 1); +lean_inc(x_59); +lean_dec(x_58); +x_60 = lean_ctor_get(x_17, 1); +lean_inc(x_60); +x_61 = l_Lean_Expr_fvarId_x21(x_9); +lean_dec(x_9); +x_62 = l_Lean_Meta_getLocalInstances(x_17, x_18, x_19, x_20, x_59); +x_63 = lean_ctor_get(x_60, 0); +lean_inc(x_63); +x_64 = lean_ctor_get(x_60, 1); +lean_inc(x_64); +lean_inc(x_60); +x_65 = lean_local_ctx_find(x_60, x_61); +if (lean_obj_tag(x_65) == 0) { -size_t x_292; lean_object* x_293; lean_object* x_294; -x_292 = lean_usize_of_nat(x_244); -lean_dec(x_244); -x_293 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__5(x_4, x_275, x_292, x_274); -x_294 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults(x_293, x_279, x_10, x_11, x_12, x_13, x_14, x_15, x_280); -return x_294; -} -} +lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; +lean_dec(x_64); +lean_dec(x_63); +x_66 = lean_ctor_get(x_62, 0); +lean_inc(x_66); +x_67 = lean_ctor_get(x_62, 1); +lean_inc(x_67); +lean_dec(x_62); +x_68 = lean_alloc_closure((void*)(l_Lean_Elab_Command_mkStructureDecl___lambda__3___boxed), 18, 11); +lean_closure_set(x_68, 0, x_5); +lean_closure_set(x_68, 1, x_4); +lean_closure_set(x_68, 2, x_8); +lean_closure_set(x_68, 3, x_54); +lean_closure_set(x_68, 4, x_11); +lean_closure_set(x_68, 5, x_12); +lean_closure_set(x_68, 6, x_13); +lean_closure_set(x_68, 7, x_7); +lean_closure_set(x_68, 8, x_50); +lean_closure_set(x_68, 9, x_35); +lean_closure_set(x_68, 10, x_34); +x_69 = l_Lean_Meta_withLCtx___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__3___rarg(x_60, x_66, x_68, x_15, x_16, x_17, x_18, x_19, x_20, x_67); +return x_69; } else { -size_t x_295; lean_object* x_296; -x_295 = lean_usize_of_nat(x_235); -lean_dec(x_235); -x_296 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__6(x_68, x_275, x_295, x_274); -lean_dec(x_68); -if (x_246 == 0) -{ -lean_object* x_297; -lean_dec(x_244); -x_297 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults(x_296, x_279, x_10, x_11, x_12, x_13, x_14, x_15, x_280); -return x_297; -} -else +uint8_t x_70; +x_70 = !lean_is_exclusive(x_60); +if (x_70 == 0) { -uint8_t x_298; -x_298 = lean_nat_dec_le(x_244, x_244); -if (x_298 == 0) +lean_object* x_71; lean_object* x_72; uint8_t x_73; +x_71 = lean_ctor_get(x_60, 1); +lean_dec(x_71); +x_72 = lean_ctor_get(x_60, 0); +lean_dec(x_72); +x_73 = !lean_is_exclusive(x_65); +if (x_73 == 0) { -lean_object* x_299; -lean_dec(x_244); -x_299 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults(x_296, x_279, x_10, x_11, x_12, x_13, x_14, x_15, x_280); -return x_299; +lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; +x_74 = lean_ctor_get(x_65, 0); +x_75 = lean_ctor_get(x_62, 0); +lean_inc(x_75); +x_76 = lean_ctor_get(x_62, 1); +lean_inc(x_76); +lean_dec(x_62); +x_77 = lean_box(0); +x_78 = l_Lean_LocalDecl_setUserName(x_74, x_77); +x_79 = l_Lean_LocalDecl_fvarId(x_78); +lean_inc(x_78); +x_80 = l_Lean_PersistentHashMap_insert___at_Lean_LocalContext_mkLocalDecl___spec__1(x_63, x_79, x_78); +x_81 = l_Lean_LocalDecl_index(x_78); +lean_ctor_set(x_65, 0, x_78); +x_82 = l_Lean_PersistentArray_set___rarg(x_64, x_81, x_65); +lean_dec(x_81); +lean_ctor_set(x_60, 1, x_82); +lean_ctor_set(x_60, 0, x_80); +x_83 = lean_alloc_closure((void*)(l_Lean_Elab_Command_mkStructureDecl___lambda__3___boxed), 18, 11); +lean_closure_set(x_83, 0, x_5); +lean_closure_set(x_83, 1, x_4); +lean_closure_set(x_83, 2, x_8); +lean_closure_set(x_83, 3, x_54); +lean_closure_set(x_83, 4, x_11); +lean_closure_set(x_83, 5, x_12); +lean_closure_set(x_83, 6, x_13); +lean_closure_set(x_83, 7, x_7); +lean_closure_set(x_83, 8, x_50); +lean_closure_set(x_83, 9, x_35); +lean_closure_set(x_83, 10, x_34); +x_84 = l_Lean_Meta_withLCtx___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__3___rarg(x_60, x_75, x_83, x_15, x_16, x_17, x_18, x_19, x_20, x_76); +return x_84; } else { -size_t x_300; lean_object* x_301; lean_object* x_302; -x_300 = lean_usize_of_nat(x_244); -lean_dec(x_244); -x_301 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__5(x_4, x_275, x_300, x_296); -x_302 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults(x_301, x_279, x_10, x_11, x_12, x_13, x_14, x_15, x_280); -return x_302; -} -} -} +lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; +x_85 = lean_ctor_get(x_65, 0); +lean_inc(x_85); +lean_dec(x_65); +x_86 = lean_ctor_get(x_62, 0); +lean_inc(x_86); +x_87 = lean_ctor_get(x_62, 1); +lean_inc(x_87); +lean_dec(x_62); +x_88 = lean_box(0); +x_89 = l_Lean_LocalDecl_setUserName(x_85, x_88); +x_90 = l_Lean_LocalDecl_fvarId(x_89); +lean_inc(x_89); +x_91 = l_Lean_PersistentHashMap_insert___at_Lean_LocalContext_mkLocalDecl___spec__1(x_63, x_90, x_89); +x_92 = l_Lean_LocalDecl_index(x_89); +x_93 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_93, 0, x_89); +x_94 = l_Lean_PersistentArray_set___rarg(x_64, x_92, x_93); +lean_dec(x_92); +lean_ctor_set(x_60, 1, x_94); +lean_ctor_set(x_60, 0, x_91); +x_95 = lean_alloc_closure((void*)(l_Lean_Elab_Command_mkStructureDecl___lambda__3___boxed), 18, 11); +lean_closure_set(x_95, 0, x_5); +lean_closure_set(x_95, 1, x_4); +lean_closure_set(x_95, 2, x_8); +lean_closure_set(x_95, 3, x_54); +lean_closure_set(x_95, 4, x_11); +lean_closure_set(x_95, 5, x_12); +lean_closure_set(x_95, 6, x_13); +lean_closure_set(x_95, 7, x_7); +lean_closure_set(x_95, 8, x_50); +lean_closure_set(x_95, 9, x_35); +lean_closure_set(x_95, 10, x_34); +x_96 = l_Lean_Meta_withLCtx___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__3___rarg(x_60, x_86, x_95, x_15, x_16, x_17, x_18, x_19, x_20, x_87); +return x_96; } } else { -lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; -lean_dec(x_274); -lean_dec(x_244); -lean_dec(x_235); -lean_dec(x_68); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -x_303 = lean_ctor_get(x_278, 0); -lean_inc(x_303); -x_304 = lean_ctor_get(x_278, 1); -lean_inc(x_304); -if (lean_is_exclusive(x_278)) { - lean_ctor_release(x_278, 0); - lean_ctor_release(x_278, 1); - x_305 = x_278; +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_dec(x_60); +x_97 = lean_ctor_get(x_65, 0); +lean_inc(x_97); +if (lean_is_exclusive(x_65)) { + lean_ctor_release(x_65, 0); + x_98 = x_65; } else { - lean_dec_ref(x_278); - x_305 = lean_box(0); + lean_dec_ref(x_65); + x_98 = lean_box(0); } -if (lean_is_scalar(x_305)) { - x_306 = lean_alloc_ctor(1, 2, 0); +x_99 = lean_ctor_get(x_62, 0); +lean_inc(x_99); +x_100 = lean_ctor_get(x_62, 1); +lean_inc(x_100); +lean_dec(x_62); +x_101 = lean_box(0); +x_102 = l_Lean_LocalDecl_setUserName(x_97, x_101); +x_103 = l_Lean_LocalDecl_fvarId(x_102); +lean_inc(x_102); +x_104 = l_Lean_PersistentHashMap_insert___at_Lean_LocalContext_mkLocalDecl___spec__1(x_63, x_103, x_102); +x_105 = l_Lean_LocalDecl_index(x_102); +if (lean_is_scalar(x_98)) { + x_106 = lean_alloc_ctor(1, 1, 0); } else { - x_306 = x_305; -} -lean_ctor_set(x_306, 0, x_303); -lean_ctor_set(x_306, 1, x_304); -return x_306; + x_106 = x_98; } +lean_ctor_set(x_106, 0, x_102); +x_107 = l_Lean_PersistentArray_set___rarg(x_64, x_105, x_106); +lean_dec(x_105); +x_108 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_108, 0, x_104); +lean_ctor_set(x_108, 1, x_107); +x_109 = lean_alloc_closure((void*)(l_Lean_Elab_Command_mkStructureDecl___lambda__3___boxed), 18, 11); +lean_closure_set(x_109, 0, x_5); +lean_closure_set(x_109, 1, x_4); +lean_closure_set(x_109, 2, x_8); +lean_closure_set(x_109, 3, x_54); +lean_closure_set(x_109, 4, x_11); +lean_closure_set(x_109, 5, x_12); +lean_closure_set(x_109, 6, x_13); +lean_closure_set(x_109, 7, x_7); +lean_closure_set(x_109, 8, x_50); +lean_closure_set(x_109, 9, x_35); +lean_closure_set(x_109, 10, x_34); +x_110 = l_Lean_Meta_withLCtx___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__3___rarg(x_108, x_99, x_109, x_15, x_16, x_17, x_18, x_19, x_20, x_100); +return x_110; } } } else { -lean_object* x_325; lean_object* x_326; lean_object* x_327; lean_object* x_328; -lean_dec(x_244); -lean_dec(x_235); -lean_dec(x_68); -lean_dec(x_67); +uint8_t x_111; +lean_dec(x_50); +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); lean_dec(x_15); -lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); -lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_5); -x_325 = lean_ctor_get(x_269, 0); -lean_inc(x_325); -x_326 = lean_ctor_get(x_269, 1); -lean_inc(x_326); -if (lean_is_exclusive(x_269)) { - lean_ctor_release(x_269, 0); - lean_ctor_release(x_269, 1); - x_327 = x_269; -} else { - lean_dec_ref(x_269); - x_327 = lean_box(0); +lean_dec(x_4); +x_111 = !lean_is_exclusive(x_58); +if (x_111 == 0) +{ +return x_58; } -if (lean_is_scalar(x_327)) { - x_328 = lean_alloc_ctor(1, 2, 0); -} else { - x_328 = x_327; +else +{ +lean_object* x_112; lean_object* x_113; lean_object* x_114; +x_112 = lean_ctor_get(x_58, 0); +x_113 = lean_ctor_get(x_58, 1); +lean_inc(x_113); +lean_inc(x_112); +lean_dec(x_58); +x_114 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_114, 0, x_112); +lean_ctor_set(x_114, 1, x_113); +return x_114; } -lean_ctor_set(x_328, 0, x_325); -lean_ctor_set(x_328, 1, x_326); -return x_328; } } else { -lean_object* x_329; lean_object* x_330; lean_object* x_331; lean_object* x_332; -lean_dec(x_257); -lean_dec(x_244); -lean_dec(x_235); -lean_dec(x_68); -lean_dec(x_67); +uint8_t x_115; +lean_dec(x_55); +lean_dec(x_50); +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); lean_dec(x_15); -lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); -lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_5); -x_329 = lean_ctor_get(x_265, 0); -lean_inc(x_329); -x_330 = lean_ctor_get(x_265, 1); -lean_inc(x_330); -if (lean_is_exclusive(x_265)) { - lean_ctor_release(x_265, 0); - lean_ctor_release(x_265, 1); - x_331 = x_265; -} else { - lean_dec_ref(x_265); - x_331 = lean_box(0); +lean_dec(x_4); +x_115 = !lean_is_exclusive(x_56); +if (x_115 == 0) +{ +return x_56; } -if (lean_is_scalar(x_331)) { - x_332 = lean_alloc_ctor(1, 2, 0); -} else { - x_332 = x_331; +else +{ +lean_object* x_116; lean_object* x_117; lean_object* x_118; +x_116 = lean_ctor_get(x_56, 0); +x_117 = lean_ctor_get(x_56, 1); +lean_inc(x_117); +lean_inc(x_116); +lean_dec(x_56); +x_118 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_118, 0, x_116); +lean_ctor_set(x_118, 1, x_117); +return x_118; } -lean_ctor_set(x_332, 0, x_329); -lean_ctor_set(x_332, 1, x_330); -return x_332; } } else { -lean_object* x_333; lean_object* x_334; lean_object* x_335; lean_object* x_336; -lean_dec(x_257); -lean_dec(x_244); -lean_dec(x_237); -lean_dec(x_235); -lean_dec(x_231); -lean_dec(x_68); -lean_dec(x_67); +uint8_t x_119; +lean_dec(x_50); +lean_free_object(x_45); +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); lean_dec(x_15); -lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); -lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_5); -x_333 = lean_ctor_get(x_261, 0); -lean_inc(x_333); -x_334 = lean_ctor_get(x_261, 1); -lean_inc(x_334); -if (lean_is_exclusive(x_261)) { - lean_ctor_release(x_261, 0); - lean_ctor_release(x_261, 1); - x_335 = x_261; -} else { - lean_dec_ref(x_261); - x_335 = lean_box(0); +lean_dec(x_4); +x_119 = !lean_is_exclusive(x_51); +if (x_119 == 0) +{ +return x_51; } -if (lean_is_scalar(x_335)) { - x_336 = lean_alloc_ctor(1, 2, 0); -} else { - x_336 = x_335; +else +{ +lean_object* x_120; lean_object* x_121; lean_object* x_122; +x_120 = lean_ctor_get(x_51, 0); +x_121 = lean_ctor_get(x_51, 1); +lean_inc(x_121); +lean_inc(x_120); +lean_dec(x_51); +x_122 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_122, 0, x_120); +lean_ctor_set(x_122, 1, x_121); +return x_122; } -lean_ctor_set(x_336, 0, x_333); -lean_ctor_set(x_336, 1, x_334); -return x_336; } } +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_45, 0); +x_124 = lean_ctor_get(x_45, 1); +lean_inc(x_124); +lean_inc(x_123); +lean_dec(x_45); +x_125 = lean_array_get_size(x_2); +lean_dec(x_2); +x_126 = lean_array_get_size(x_35); +lean_inc(x_20); +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_126); +lean_inc(x_34); +lean_inc(x_9); +lean_inc(x_8); +x_127 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkInductiveType(x_8, x_9, x_34, x_125, x_126, x_123, x_37, x_15, x_16, x_17, x_18, x_19, x_20, x_124); +if (lean_obj_tag(x_127) == 0) +{ +lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; +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_box(0); +x_131 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_131, 0, x_128); +lean_ctor_set(x_131, 1, x_130); +lean_inc(x_126); +lean_inc(x_34); +x_132 = lean_alloc_ctor(6, 3, 1); +lean_ctor_set(x_132, 0, x_34); +lean_ctor_set(x_132, 1, x_126); +lean_ctor_set(x_132, 2, x_131); +lean_ctor_set_uint8(x_132, sizeof(void*)*3, x_10); +lean_inc(x_20); +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_132); +x_133 = l_Lean_Elab_Term_ensureNoUnassignedMVars(x_132, x_15, x_16, x_17, x_18, x_19, x_20, x_129); +if (lean_obj_tag(x_133) == 0) +{ +lean_object* x_134; lean_object* x_135; +x_134 = lean_ctor_get(x_133, 1); +lean_inc(x_134); +lean_dec(x_133); +lean_inc(x_20); +lean_inc(x_19); +x_135 = l_Lean_addDecl(x_132, x_19, x_20, x_134); +if (lean_obj_tag(x_135) == 0) +{ +lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; +x_136 = lean_ctor_get(x_135, 1); +lean_inc(x_136); +lean_dec(x_135); +x_137 = lean_ctor_get(x_17, 1); +lean_inc(x_137); +x_138 = l_Lean_Expr_fvarId_x21(x_9); +lean_dec(x_9); +x_139 = l_Lean_Meta_getLocalInstances(x_17, x_18, x_19, x_20, x_136); +x_140 = lean_ctor_get(x_137, 0); +lean_inc(x_140); +x_141 = lean_ctor_get(x_137, 1); +lean_inc(x_141); +lean_inc(x_137); +x_142 = lean_local_ctx_find(x_137, x_138); +if (lean_obj_tag(x_142) == 0) +{ +lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; +lean_dec(x_141); +lean_dec(x_140); +x_143 = lean_ctor_get(x_139, 0); +lean_inc(x_143); +x_144 = lean_ctor_get(x_139, 1); +lean_inc(x_144); +lean_dec(x_139); +x_145 = lean_alloc_closure((void*)(l_Lean_Elab_Command_mkStructureDecl___lambda__3___boxed), 18, 11); +lean_closure_set(x_145, 0, x_5); +lean_closure_set(x_145, 1, x_4); +lean_closure_set(x_145, 2, x_8); +lean_closure_set(x_145, 3, x_130); +lean_closure_set(x_145, 4, x_11); +lean_closure_set(x_145, 5, x_12); +lean_closure_set(x_145, 6, x_13); +lean_closure_set(x_145, 7, x_7); +lean_closure_set(x_145, 8, x_126); +lean_closure_set(x_145, 9, x_35); +lean_closure_set(x_145, 10, x_34); +x_146 = l_Lean_Meta_withLCtx___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__3___rarg(x_137, x_143, x_145, x_15, x_16, x_17, x_18, x_19, x_20, x_144); +return x_146; } else { -lean_object* x_351; lean_object* x_352; lean_object* x_353; lean_object* x_354; -lean_dec(x_244); -lean_dec(x_237); -lean_dec(x_235); -lean_dec(x_231); -lean_dec(x_68); -lean_dec(x_67); -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_7); -lean_dec(x_6); -lean_dec(x_5); -x_351 = lean_ctor_get(x_255, 0); -lean_inc(x_351); -x_352 = lean_ctor_get(x_255, 1); -lean_inc(x_352); -if (lean_is_exclusive(x_255)) { - lean_ctor_release(x_255, 0); - lean_ctor_release(x_255, 1); - x_353 = x_255; +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; +if (lean_is_exclusive(x_137)) { + lean_ctor_release(x_137, 0); + lean_ctor_release(x_137, 1); + x_147 = x_137; } else { - lean_dec_ref(x_255); - x_353 = lean_box(0); + lean_dec_ref(x_137); + x_147 = lean_box(0); } -if (lean_is_scalar(x_353)) { - x_354 = lean_alloc_ctor(1, 2, 0); +x_148 = lean_ctor_get(x_142, 0); +lean_inc(x_148); +if (lean_is_exclusive(x_142)) { + lean_ctor_release(x_142, 0); + x_149 = x_142; } else { - x_354 = x_353; -} -lean_ctor_set(x_354, 0, x_351); -lean_ctor_set(x_354, 1, x_352); -return x_354; + lean_dec_ref(x_142); + x_149 = lean_box(0); } -} -else -{ -lean_object* x_355; lean_object* x_356; lean_object* x_357; lean_object* x_358; -lean_dec(x_244); -lean_dec(x_237); -lean_dec(x_235); -lean_dec(x_231); -lean_dec(x_68); -lean_dec(x_67); -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_7); -lean_dec(x_6); -lean_dec(x_5); -x_355 = lean_ctor_get(x_253, 0); -lean_inc(x_355); -x_356 = lean_ctor_get(x_253, 1); -lean_inc(x_356); -if (lean_is_exclusive(x_253)) { - lean_ctor_release(x_253, 0); - lean_ctor_release(x_253, 1); - x_357 = x_253; +x_150 = lean_ctor_get(x_139, 0); +lean_inc(x_150); +x_151 = lean_ctor_get(x_139, 1); +lean_inc(x_151); +lean_dec(x_139); +x_152 = lean_box(0); +x_153 = l_Lean_LocalDecl_setUserName(x_148, x_152); +x_154 = l_Lean_LocalDecl_fvarId(x_153); +lean_inc(x_153); +x_155 = l_Lean_PersistentHashMap_insert___at_Lean_LocalContext_mkLocalDecl___spec__1(x_140, x_154, x_153); +x_156 = l_Lean_LocalDecl_index(x_153); +if (lean_is_scalar(x_149)) { + x_157 = lean_alloc_ctor(1, 1, 0); } else { - lean_dec_ref(x_253); - x_357 = lean_box(0); + x_157 = x_149; } -if (lean_is_scalar(x_357)) { - x_358 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_157, 0, x_153); +x_158 = l_Lean_PersistentArray_set___rarg(x_141, x_156, x_157); +lean_dec(x_156); +if (lean_is_scalar(x_147)) { + x_159 = lean_alloc_ctor(0, 2, 0); } else { - x_358 = x_357; + x_159 = x_147; } -lean_ctor_set(x_358, 0, x_355); -lean_ctor_set(x_358, 1, x_356); -return x_358; +lean_ctor_set(x_159, 0, x_155); +lean_ctor_set(x_159, 1, x_158); +x_160 = lean_alloc_closure((void*)(l_Lean_Elab_Command_mkStructureDecl___lambda__3___boxed), 18, 11); +lean_closure_set(x_160, 0, x_5); +lean_closure_set(x_160, 1, x_4); +lean_closure_set(x_160, 2, x_8); +lean_closure_set(x_160, 3, x_130); +lean_closure_set(x_160, 4, x_11); +lean_closure_set(x_160, 5, x_12); +lean_closure_set(x_160, 6, x_13); +lean_closure_set(x_160, 7, x_7); +lean_closure_set(x_160, 8, x_126); +lean_closure_set(x_160, 9, x_35); +lean_closure_set(x_160, 10, x_34); +x_161 = l_Lean_Meta_withLCtx___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__3___rarg(x_159, x_150, x_160, x_15, x_16, x_17, x_18, x_19, x_20, x_151); +return x_161; } } else { -lean_object* x_359; lean_object* x_360; lean_object* x_361; lean_object* x_362; -lean_dec(x_244); -lean_dec(x_237); -lean_dec(x_235); -lean_dec(x_231); -lean_dec(x_68); -lean_dec(x_67); +lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; +lean_dec(x_126); +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); lean_dec(x_15); -lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); -lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); lean_dec(x_5); -x_359 = lean_ctor_get(x_251, 0); -lean_inc(x_359); -x_360 = lean_ctor_get(x_251, 1); -lean_inc(x_360); -if (lean_is_exclusive(x_251)) { - lean_ctor_release(x_251, 0); - lean_ctor_release(x_251, 1); - x_361 = x_251; +lean_dec(x_4); +x_162 = lean_ctor_get(x_135, 0); +lean_inc(x_162); +x_163 = lean_ctor_get(x_135, 1); +lean_inc(x_163); +if (lean_is_exclusive(x_135)) { + lean_ctor_release(x_135, 0); + lean_ctor_release(x_135, 1); + x_164 = x_135; } else { - lean_dec_ref(x_251); - x_361 = lean_box(0); + lean_dec_ref(x_135); + x_164 = lean_box(0); } -if (lean_is_scalar(x_361)) { - x_362 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_164)) { + x_165 = lean_alloc_ctor(1, 2, 0); } else { - x_362 = x_361; -} -lean_ctor_set(x_362, 0, x_359); -lean_ctor_set(x_362, 1, x_360); -return x_362; + x_165 = x_164; } +lean_ctor_set(x_165, 0, x_162); +lean_ctor_set(x_165, 1, x_163); +return x_165; } } else { -lean_object* x_371; lean_object* x_372; lean_object* x_373; lean_object* x_374; -lean_dec(x_237); -lean_dec(x_235); -lean_dec(x_231); -lean_dec(x_68); -lean_dec(x_67); +lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; +lean_dec(x_132); +lean_dec(x_126); +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); lean_dec(x_15); -lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); -lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); lean_dec(x_5); -x_371 = lean_ctor_get(x_242, 0); -lean_inc(x_371); -x_372 = lean_ctor_get(x_242, 1); -lean_inc(x_372); -if (lean_is_exclusive(x_242)) { - lean_ctor_release(x_242, 0); - lean_ctor_release(x_242, 1); - x_373 = x_242; +lean_dec(x_4); +x_166 = lean_ctor_get(x_133, 0); +lean_inc(x_166); +x_167 = lean_ctor_get(x_133, 1); +lean_inc(x_167); +if (lean_is_exclusive(x_133)) { + lean_ctor_release(x_133, 0); + lean_ctor_release(x_133, 1); + x_168 = x_133; } else { - lean_dec_ref(x_242); - x_373 = lean_box(0); + lean_dec_ref(x_133); + x_168 = lean_box(0); } -if (lean_is_scalar(x_373)) { - x_374 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_168)) { + x_169 = lean_alloc_ctor(1, 2, 0); } else { - x_374 = x_373; + x_169 = x_168; } -lean_ctor_set(x_374, 0, x_371); -lean_ctor_set(x_374, 1, x_372); -return x_374; +lean_ctor_set(x_169, 0, x_166); +lean_ctor_set(x_169, 1, x_167); +return x_169; } } else { -lean_object* x_375; lean_object* x_376; lean_object* x_377; lean_object* x_378; -lean_dec(x_239); -lean_dec(x_237); -lean_dec(x_235); -lean_dec(x_231); -lean_dec(x_68); -lean_dec(x_67); +lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; +lean_dec(x_126); +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); lean_dec(x_15); -lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); -lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); lean_dec(x_5); -x_375 = lean_ctor_get(x_240, 0); -lean_inc(x_375); -x_376 = lean_ctor_get(x_240, 1); -lean_inc(x_376); -if (lean_is_exclusive(x_240)) { - lean_ctor_release(x_240, 0); - lean_ctor_release(x_240, 1); - x_377 = x_240; +lean_dec(x_4); +x_170 = lean_ctor_get(x_127, 0); +lean_inc(x_170); +x_171 = lean_ctor_get(x_127, 1); +lean_inc(x_171); +if (lean_is_exclusive(x_127)) { + lean_ctor_release(x_127, 0); + lean_ctor_release(x_127, 1); + x_172 = x_127; } else { - lean_dec_ref(x_240); - x_377 = lean_box(0); + lean_dec_ref(x_127); + x_172 = lean_box(0); } -if (lean_is_scalar(x_377)) { - x_378 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_172)) { + x_173 = lean_alloc_ctor(1, 2, 0); } else { - x_378 = x_377; + x_173 = x_172; } -lean_ctor_set(x_378, 0, x_375); -lean_ctor_set(x_378, 1, x_376); -return x_378; +lean_ctor_set(x_173, 0, x_170); +lean_ctor_set(x_173, 1, x_171); +return x_173; } } } else { -uint8_t x_379; -lean_dec(x_70); -lean_dec(x_68); -lean_dec(x_67); +uint8_t x_174; +lean_dec(x_37); +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); lean_dec(x_15); -lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); -lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); lean_dec(x_5); -x_379 = !lean_is_exclusive(x_75); -if (x_379 == 0) +lean_dec(x_4); +lean_dec(x_2); +x_174 = !lean_is_exclusive(x_42); +if (x_174 == 0) { -return x_75; +return x_42; } else { -lean_object* x_380; lean_object* x_381; lean_object* x_382; -x_380 = lean_ctor_get(x_75, 0); -x_381 = lean_ctor_get(x_75, 1); -lean_inc(x_381); -lean_inc(x_380); -lean_dec(x_75); -x_382 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_382, 0, x_380); -lean_ctor_set(x_382, 1, x_381); -return x_382; +lean_object* x_175; lean_object* x_176; lean_object* x_177; +x_175 = lean_ctor_get(x_42, 0); +x_176 = lean_ctor_get(x_42, 1); +lean_inc(x_176); +lean_inc(x_175); +lean_dec(x_42); +x_177 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_177, 0, x_175); +lean_ctor_set(x_177, 1, x_176); +return x_177; } } } else { -uint8_t x_383; -lean_dec(x_68); -lean_dec(x_67); +uint8_t x_178; +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); lean_dec(x_15); -lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); -lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); lean_dec(x_1); -x_383 = !lean_is_exclusive(x_69); -if (x_383 == 0) +x_178 = !lean_is_exclusive(x_36); +if (x_178 == 0) { -return x_69; +return x_36; } else { -lean_object* x_384; lean_object* x_385; lean_object* x_386; -x_384 = lean_ctor_get(x_69, 0); -x_385 = lean_ctor_get(x_69, 1); -lean_inc(x_385); -lean_inc(x_384); -lean_dec(x_69); -x_386 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_386, 0, x_384); -lean_ctor_set(x_386, 1, x_385); -return x_386; +lean_object* x_179; lean_object* x_180; lean_object* x_181; +x_179 = lean_ctor_get(x_36, 0); +x_180 = lean_ctor_get(x_36, 1); +lean_inc(x_180); +lean_inc(x_179); +lean_dec(x_36); +x_181 = lean_alloc_ctor(1, 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_387; +uint8_t x_182; +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); lean_dec(x_15); -lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); -lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); +lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_387 = !lean_is_exclusive(x_17); -if (x_387 == 0) +x_182 = !lean_is_exclusive(x_22); +if (x_182 == 0) { -return x_17; +return x_22; } else { -lean_object* x_388; lean_object* x_389; lean_object* x_390; -x_388 = lean_ctor_get(x_17, 0); -x_389 = lean_ctor_get(x_17, 1); -lean_inc(x_389); -lean_inc(x_388); -lean_dec(x_17); -x_390 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_390, 0, x_388); -lean_ctor_set(x_390, 1, x_389); -return x_390; -} -} +lean_object* x_183; lean_object* x_184; lean_object* x_185; +x_183 = lean_ctor_get(x_22, 0); +x_184 = lean_ctor_get(x_22, 1); +lean_inc(x_184); +lean_inc(x_183); +lean_dec(x_22); +x_185 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_185, 0, x_183); +lean_ctor_set(x_185, 1, x_184); +return x_185; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__4___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__5; -x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__4; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__4___closed__2() { +static lean_object* _init_l_Lean_Elab_Command_mkStructureDecl___lambda__5___closed__1() { _start: { lean_object* x_1; @@ -32752,458 +31998,469 @@ x_1 = lean_mk_string_unchecked("type: ", 6, 6); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__4___closed__3() { +static lean_object* _init_l_Lean_Elab_Command_mkStructureDecl___lambda__5___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__4___closed__2; +x_1 = l_Lean_Elab_Command_mkStructureDecl___lambda__5___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___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, uint8_t x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19, lean_object* x_20, lean_object* x_21, lean_object* x_22) { _start: { -lean_object* x_17; -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); +lean_object* x_23; +lean_inc(x_21); +lean_inc(x_20); +lean_inc(x_19); +lean_inc(x_18); lean_inc(x_3); -x_17 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_levelMVarToParam(x_9, x_1, x_2, x_3, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_17) == 0) +x_23 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_levelMVarToParam(x_15, x_1, x_2, x_3, x_16, x_17, x_18, x_19, x_20, x_21, x_22); +if (lean_obj_tag(x_23) == 0) { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; lean_object* x_63; uint8_t x_64; lean_object* x_65; lean_object* x_66; -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_51 = lean_ctor_get(x_14, 0); -lean_inc(x_51); -x_52 = lean_ctor_get(x_14, 1); -lean_inc(x_52); -x_53 = lean_ctor_get(x_14, 2); -lean_inc(x_53); -x_54 = lean_ctor_get(x_14, 3); -lean_inc(x_54); -x_55 = lean_ctor_get(x_14, 4); -lean_inc(x_55); -x_56 = lean_ctor_get(x_14, 5); +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; uint8_t x_67; lean_object* x_68; uint8_t x_69; lean_object* x_70; lean_object* x_71; +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_56 = lean_ctor_get(x_20, 0); lean_inc(x_56); -x_57 = lean_ctor_get(x_14, 6); +x_57 = lean_ctor_get(x_20, 1); lean_inc(x_57); -x_58 = lean_ctor_get(x_14, 7); +x_58 = lean_ctor_get(x_20, 2); lean_inc(x_58); -x_59 = lean_ctor_get(x_14, 8); +x_59 = lean_ctor_get(x_20, 3); lean_inc(x_59); -x_60 = lean_ctor_get(x_14, 9); +x_60 = lean_ctor_get(x_20, 4); lean_inc(x_60); -x_61 = lean_ctor_get(x_14, 10); +x_61 = lean_ctor_get(x_20, 5); lean_inc(x_61); -x_62 = lean_ctor_get_uint8(x_14, sizeof(void*)*12); -x_63 = lean_ctor_get(x_14, 11); +x_62 = lean_ctor_get(x_20, 6); +lean_inc(x_62); +x_63 = lean_ctor_get(x_20, 7); lean_inc(x_63); -x_64 = lean_ctor_get_uint8(x_14, sizeof(void*)*12 + 1); -x_65 = l_Lean_replaceRef(x_5, x_56); -lean_dec(x_56); -x_66 = lean_alloc_ctor(0, 12, 2); -lean_ctor_set(x_66, 0, x_51); -lean_ctor_set(x_66, 1, x_52); -lean_ctor_set(x_66, 2, x_53); -lean_ctor_set(x_66, 3, x_54); -lean_ctor_set(x_66, 4, x_55); -lean_ctor_set(x_66, 5, x_65); -lean_ctor_set(x_66, 6, x_57); -lean_ctor_set(x_66, 7, x_58); -lean_ctor_set(x_66, 8, x_59); -lean_ctor_set(x_66, 9, x_60); -lean_ctor_set(x_66, 10, x_61); -lean_ctor_set(x_66, 11, x_63); -lean_ctor_set_uint8(x_66, sizeof(void*)*12, x_62); -lean_ctor_set_uint8(x_66, sizeof(void*)*12 + 1, x_64); -if (lean_obj_tag(x_3) == 0) -{ -lean_object* x_67; -lean_inc(x_15); +x_64 = lean_ctor_get(x_20, 8); +lean_inc(x_64); +x_65 = lean_ctor_get(x_20, 9); +lean_inc(x_65); +x_66 = lean_ctor_get(x_20, 10); lean_inc(x_66); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_10); -lean_inc(x_8); -x_67 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getResultUniverse(x_8, x_10, x_11, x_12, x_13, x_66, x_15, x_19); -if (lean_obj_tag(x_67) == 0) -{ -lean_object* x_68; lean_object* x_69; lean_object* x_70; -x_68 = lean_ctor_get(x_67, 0); +x_67 = lean_ctor_get_uint8(x_20, sizeof(void*)*12); +x_68 = lean_ctor_get(x_20, 11); lean_inc(x_68); -x_69 = lean_ctor_get(x_67, 1); -lean_inc(x_69); -lean_dec(x_67); -lean_inc(x_10); -x_70 = l_Lean_Elab_Command_checkResultingUniverse(x_68, x_10, x_11, x_12, x_13, x_66, x_15, x_69); -lean_dec(x_66); -if (lean_obj_tag(x_70) == 0) +x_69 = lean_ctor_get_uint8(x_20, sizeof(void*)*12 + 1); +x_70 = l_Lean_replaceRef(x_11, x_61); +lean_dec(x_61); +x_71 = lean_alloc_ctor(0, 12, 2); +lean_ctor_set(x_71, 0, x_56); +lean_ctor_set(x_71, 1, x_57); +lean_ctor_set(x_71, 2, x_58); +lean_ctor_set(x_71, 3, x_59); +lean_ctor_set(x_71, 4, x_60); +lean_ctor_set(x_71, 5, x_70); +lean_ctor_set(x_71, 6, x_62); +lean_ctor_set(x_71, 7, x_63); +lean_ctor_set(x_71, 8, x_64); +lean_ctor_set(x_71, 9, x_65); +lean_ctor_set(x_71, 10, x_66); +lean_ctor_set(x_71, 11, x_68); +lean_ctor_set_uint8(x_71, sizeof(void*)*12, x_67); +lean_ctor_set_uint8(x_71, sizeof(void*)*12 + 1, x_69); +if (lean_obj_tag(x_3) == 0) { -lean_object* x_71; -x_71 = lean_ctor_get(x_70, 1); +lean_object* x_72; +lean_inc(x_21); lean_inc(x_71); -lean_dec(x_70); -x_20 = x_8; -x_21 = x_71; -goto block_50; +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_16); +lean_inc(x_14); +x_72 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getResultUniverse(x_14, x_16, x_17, x_18, x_19, x_71, x_21, x_25); +if (lean_obj_tag(x_72) == 0) +{ +lean_object* x_73; lean_object* x_74; lean_object* x_75; +x_73 = lean_ctor_get(x_72, 0); +lean_inc(x_73); +x_74 = lean_ctor_get(x_72, 1); +lean_inc(x_74); +lean_dec(x_72); +lean_inc(x_16); +x_75 = l_Lean_Elab_Command_checkResultingUniverse(x_73, x_16, x_17, x_18, x_19, x_71, x_21, x_74); +lean_dec(x_71); +if (lean_obj_tag(x_75) == 0) +{ +lean_object* x_76; +x_76 = lean_ctor_get(x_75, 1); +lean_inc(x_76); +lean_dec(x_75); +x_26 = x_14; +x_27 = x_76; +goto block_55; } else { -uint8_t x_72; +uint8_t x_77; +lean_dec(x_24); +lean_dec(x_21); +lean_dec(x_20); +lean_dec(x_19); lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); -lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_72 = !lean_is_exclusive(x_70); -if (x_72 == 0) +x_77 = !lean_is_exclusive(x_75); +if (x_77 == 0) { -return x_70; +return x_75; } else { -lean_object* x_73; lean_object* x_74; lean_object* x_75; -x_73 = lean_ctor_get(x_70, 0); -x_74 = lean_ctor_get(x_70, 1); -lean_inc(x_74); -lean_inc(x_73); -lean_dec(x_70); -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_78; lean_object* x_79; lean_object* x_80; +x_78 = lean_ctor_get(x_75, 0); +x_79 = lean_ctor_get(x_75, 1); +lean_inc(x_79); +lean_inc(x_78); +lean_dec(x_75); +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_76; -lean_dec(x_66); +uint8_t x_81; +lean_dec(x_71); +lean_dec(x_24); +lean_dec(x_21); +lean_dec(x_20); +lean_dec(x_19); lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); -lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_76 = !lean_is_exclusive(x_67); -if (x_76 == 0) +x_81 = !lean_is_exclusive(x_72); +if (x_81 == 0) { -return x_67; +return x_72; } else { -lean_object* x_77; lean_object* x_78; lean_object* x_79; -x_77 = lean_ctor_get(x_67, 0); -x_78 = lean_ctor_get(x_67, 1); -lean_inc(x_78); -lean_inc(x_77); -lean_dec(x_67); -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_82; lean_object* x_83; lean_object* x_84; +x_82 = lean_ctor_get(x_72, 0); +x_83 = lean_ctor_get(x_72, 1); +lean_inc(x_83); +lean_inc(x_82); +lean_dec(x_72); +x_84 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_84, 0, x_82); +lean_ctor_set(x_84, 1, x_83); +return x_84; } } } else { -lean_object* x_80; +lean_object* x_85; lean_dec(x_3); -lean_inc(x_15); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -x_80 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse(x_18, x_8, x_10, x_11, x_12, x_13, x_66, x_15, x_19); -if (lean_obj_tag(x_80) == 0) +lean_inc(x_21); +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +x_85 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse(x_24, x_14, x_16, x_17, x_18, x_19, x_71, x_21, x_25); +if (lean_obj_tag(x_85) == 0) { -lean_object* x_81; lean_object* x_82; -x_81 = lean_ctor_get(x_80, 0); -lean_inc(x_81); -x_82 = lean_ctor_get(x_80, 1); -lean_inc(x_82); -lean_dec(x_80); -x_20 = x_81; -x_21 = x_82; -goto block_50; +lean_object* x_86; lean_object* x_87; +x_86 = lean_ctor_get(x_85, 0); +lean_inc(x_86); +x_87 = lean_ctor_get(x_85, 1); +lean_inc(x_87); +lean_dec(x_85); +x_26 = x_86; +x_27 = x_87; +goto block_55; } else { -uint8_t x_83; +uint8_t x_88; +lean_dec(x_24); +lean_dec(x_21); +lean_dec(x_20); +lean_dec(x_19); lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); lean_dec(x_15); -lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); -lean_dec(x_10); lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_83 = !lean_is_exclusive(x_80); -if (x_83 == 0) +x_88 = !lean_is_exclusive(x_85); +if (x_88 == 0) { -return x_80; +return x_85; } else { -lean_object* x_84; lean_object* x_85; lean_object* x_86; -x_84 = lean_ctor_get(x_80, 0); -x_85 = lean_ctor_get(x_80, 1); -lean_inc(x_85); -lean_inc(x_84); -lean_dec(x_80); -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_89; lean_object* x_90; lean_object* x_91; +x_89 = lean_ctor_get(x_85, 0); +x_90 = lean_ctor_get(x_85, 1); +lean_inc(x_90); +lean_inc(x_89); +lean_dec(x_85); +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; } } } -block_50: +block_55: { -lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; -x_22 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__4___closed__1; -x_23 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_22, x_10, x_11, x_12, x_13, x_14, x_15, x_21); -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -x_25 = lean_unbox(x_24); -lean_dec(x_24); -if (x_25 == 0) +lean_object* x_28; lean_object* x_29; uint8_t x_30; +lean_inc(x_4); +x_28 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_4, x_16, x_17, x_18, x_19, x_20, x_21, x_27); +x_29 = lean_ctor_get(x_28, 0); +lean_inc(x_29); +x_30 = lean_unbox(x_29); +lean_dec(x_29); +if (x_30 == 0) { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_23, 1); -lean_inc(x_26); -lean_dec(x_23); -x_27 = lean_box(0); -x_28 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__3(x_20, x_9, x_1, x_18, x_4, x_5, x_6, x_7, x_27, x_10, x_11, x_12, x_13, x_14, x_15, x_26); -lean_dec(x_18); -return x_28; +lean_object* x_31; lean_object* x_32; lean_object* x_33; +lean_dec(x_4); +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_Elab_Command_mkStructureDecl___lambda__4(x_26, x_15, x_1, x_24, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_32, x_16, x_17, x_18, x_19, x_20, x_21, x_31); +return x_33; } else { -uint8_t x_29; -x_29 = !lean_is_exclusive(x_23); -if (x_29 == 0) +uint8_t x_34; +x_34 = !lean_is_exclusive(x_28); +if (x_34 == 0) { -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_30 = lean_ctor_get(x_23, 1); -x_31 = lean_ctor_get(x_23, 0); -lean_dec(x_31); -lean_inc(x_20); -x_32 = l_Lean_MessageData_ofExpr(x_20); -x_33 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__4___closed__3; -lean_ctor_set_tag(x_23, 7); -lean_ctor_set(x_23, 1, x_32); -lean_ctor_set(x_23, 0, x_33); -x_34 = l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__4; -x_35 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_35, 0, x_23); -lean_ctor_set(x_35, 1, x_34); -x_36 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_22, x_35, x_10, x_11, x_12, x_13, x_14, x_15, x_30); -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_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_28, 1); +x_36 = lean_ctor_get(x_28, 0); lean_dec(x_36); -x_39 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__3(x_20, x_9, x_1, x_18, x_4, x_5, x_6, x_7, x_37, x_10, x_11, x_12, x_13, x_14, x_15, x_38); -lean_dec(x_37); -lean_dec(x_18); -return x_39; +lean_inc(x_26); +x_37 = l_Lean_MessageData_ofExpr(x_26); +x_38 = l_Lean_Elab_Command_mkStructureDecl___lambda__5___closed__2; +lean_ctor_set_tag(x_28, 7); +lean_ctor_set(x_28, 1, x_37); +lean_ctor_set(x_28, 0, x_38); +x_39 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3; +x_40 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_40, 0, x_28); +lean_ctor_set(x_40, 1, x_39); +x_41 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_4, x_40, x_16, x_17, x_18, x_19, x_20, x_21, x_35); +x_42 = lean_ctor_get(x_41, 0); +lean_inc(x_42); +x_43 = lean_ctor_get(x_41, 1); +lean_inc(x_43); +lean_dec(x_41); +x_44 = l_Lean_Elab_Command_mkStructureDecl___lambda__4(x_26, x_15, x_1, x_24, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_42, x_16, x_17, x_18, x_19, x_20, x_21, x_43); +lean_dec(x_42); +return x_44; } else { -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_40 = lean_ctor_get(x_23, 1); -lean_inc(x_40); -lean_dec(x_23); -lean_inc(x_20); -x_41 = l_Lean_MessageData_ofExpr(x_20); -x_42 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__4___closed__3; -x_43 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_43, 0, x_42); -lean_ctor_set(x_43, 1, x_41); -x_44 = l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__4; -x_45 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_45, 0, x_43); -lean_ctor_set(x_45, 1, x_44); -x_46 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_22, x_45, x_10, x_11, x_12, x_13, x_14, x_15, x_40); -x_47 = lean_ctor_get(x_46, 0); -lean_inc(x_47); -x_48 = lean_ctor_get(x_46, 1); -lean_inc(x_48); -lean_dec(x_46); -x_49 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__3(x_20, x_9, x_1, x_18, x_4, x_5, x_6, x_7, x_47, x_10, x_11, x_12, x_13, x_14, x_15, x_48); -lean_dec(x_47); -lean_dec(x_18); -return x_49; +lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_45 = lean_ctor_get(x_28, 1); +lean_inc(x_45); +lean_dec(x_28); +lean_inc(x_26); +x_46 = l_Lean_MessageData_ofExpr(x_26); +x_47 = l_Lean_Elab_Command_mkStructureDecl___lambda__5___closed__2; +x_48 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_48, 0, x_47); +lean_ctor_set(x_48, 1, x_46); +x_49 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3; +x_50 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_50, 0, x_48); +lean_ctor_set(x_50, 1, x_49); +x_51 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_4, x_50, x_16, x_17, x_18, x_19, x_20, x_21, x_45); +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_Elab_Command_mkStructureDecl___lambda__4(x_26, x_15, x_1, x_24, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_52, x_16, x_17, x_18, x_19, x_20, x_21, x_53); +lean_dec(x_52); +return x_54; } } } } else { -uint8_t x_87; +uint8_t x_92; +lean_dec(x_21); +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); -lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_87 = !lean_is_exclusive(x_17); -if (x_87 == 0) +x_92 = !lean_is_exclusive(x_23); +if (x_92 == 0) { -return x_17; +return x_23; } else { -lean_object* x_88; lean_object* x_89; lean_object* x_90; -x_88 = lean_ctor_get(x_17, 0); -x_89 = lean_ctor_get(x_17, 1); -lean_inc(x_89); -lean_inc(x_88); -lean_dec(x_17); -x_90 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_90, 0, x_88); -lean_ctor_set(x_90, 1, x_89); -return x_90; +lean_object* x_93; lean_object* x_94; lean_object* x_95; +x_93 = lean_ctor_get(x_23, 0); +x_94 = lean_ctor_get(x_23, 1); +lean_inc(x_94); +lean_inc(x_93); +lean_dec(x_23); +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_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, uint8_t x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, 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: { -uint8_t x_14; uint8_t x_15; lean_object* x_16; -x_14 = 1; -x_15 = 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_16 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_14, x_15, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_16) == 0) +uint8_t x_21; +x_21 = !lean_is_exclusive(x_18); +if (x_21 == 0) { -lean_object* x_17; lean_object* x_18; -x_17 = lean_ctor_get(x_16, 1); +lean_object* x_22; lean_object* x_23; uint8_t x_24; uint8_t x_25; lean_object* x_26; +x_22 = lean_ctor_get(x_18, 5); +x_23 = l_Lean_replaceRef(x_1, x_22); +lean_dec(x_22); +lean_ctor_set(x_18, 5, x_23); +x_24 = 1; +x_25 = 0; +lean_inc(x_19); +lean_inc(x_18); lean_inc(x_17); -lean_dec(x_16); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_7); -lean_inc(x_1); -x_18 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getResultUniverse(x_1, x_7, x_8, x_9, x_10, x_11, x_12, x_17); -if (lean_obj_tag(x_18) == 0) +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +x_26 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_24, x_25, x_14, x_15, x_16, x_17, x_18, x_19, x_20); +if (lean_obj_tag(x_26) == 0) { -lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_19 = lean_ctor_get(x_18, 0); +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_27 = lean_ctor_get(x_26, 1); +lean_inc(x_27); +lean_dec(x_26); +x_28 = lean_ctor_get(x_2, 5); +lean_inc(x_28); +x_29 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_28, x_14, x_15, x_16, x_17, x_18, x_19, x_27); +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_19); -x_20 = lean_ctor_get(x_18, 1); -lean_inc(x_20); -lean_dec(x_18); -lean_inc(x_7); -x_21 = l_Lean_Elab_Command_shouldInferResultUniverse(x_19, x_7, x_8, x_9, x_10, x_11, x_12, x_20); -if (lean_obj_tag(x_21) == 0) +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_14); +lean_inc(x_30); +x_32 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getResultUniverse(x_30, x_14, x_15, x_16, x_17, x_18, x_19, x_31); +if (lean_obj_tag(x_32) == 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_ctor_get(x_21, 0); -lean_inc(x_22); -x_23 = lean_ctor_get(x_21, 1); -lean_inc(x_23); -lean_dec(x_21); -x_24 = lean_ctor_get(x_2, 5); -lean_inc(x_24); -x_25 = lean_ctor_get(x_2, 6); -lean_inc(x_25); -lean_inc(x_6); -lean_inc(x_25); -x_26 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__4___boxed), 16, 8); -lean_closure_set(x_26, 0, x_25); -lean_closure_set(x_26, 1, x_6); -lean_closure_set(x_26, 2, x_22); -lean_closure_set(x_26, 3, x_2); -lean_closure_set(x_26, 4, x_3); -lean_closure_set(x_26, 5, x_4); -lean_closure_set(x_26, 6, x_5); -lean_closure_set(x_26, 7, x_1); -x_27 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withUsed___rarg(x_24, x_25, x_6, x_26, x_7, x_8, x_9, x_10, x_11, x_12, x_23); -lean_dec(x_6); -lean_dec(x_25); -lean_dec(x_24); -return x_27; -} -else +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); +lean_inc(x_14); +x_35 = l_Lean_Elab_Command_shouldInferResultUniverse(x_33, x_14, x_15, x_16, x_17, x_18, x_19, x_34); +if (lean_obj_tag(x_35) == 0) { -uint8_t x_28; -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_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); +lean_dec(x_35); +x_38 = lean_box(x_9); +lean_inc(x_13); +lean_inc(x_3); +x_39 = lean_alloc_closure((void*)(l_Lean_Elab_Command_mkStructureDecl___lambda__5___boxed), 22, 14); +lean_closure_set(x_39, 0, x_3); +lean_closure_set(x_39, 1, x_13); +lean_closure_set(x_39, 2, x_36); +lean_closure_set(x_39, 3, x_4); +lean_closure_set(x_39, 4, x_2); +lean_closure_set(x_39, 5, x_5); +lean_closure_set(x_39, 6, x_6); +lean_closure_set(x_39, 7, x_7); +lean_closure_set(x_39, 8, x_8); +lean_closure_set(x_39, 9, x_38); +lean_closure_set(x_39, 10, x_1); +lean_closure_set(x_39, 11, x_10); +lean_closure_set(x_39, 12, x_11); +lean_closure_set(x_39, 13, x_30); +x_40 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withUsed___rarg(x_12, x_3, x_13, x_39, x_14, x_15, x_16, x_17, x_18, x_19, x_37); +lean_dec(x_13); lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_28 = !lean_is_exclusive(x_21); -if (x_28 == 0) -{ -return x_21; -} -else -{ -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_21, 0); -x_30 = lean_ctor_get(x_21, 1); -lean_inc(x_30); -lean_inc(x_29); -lean_dec(x_21); -x_31 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_31, 0, x_29); -lean_ctor_set(x_31, 1, x_30); -return x_31; -} -} +return x_40; } else { -uint8_t x_32; -lean_dec(x_12); +uint8_t x_41; +lean_dec(x_30); +lean_dec(x_18); +lean_dec(x_19); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); lean_dec(x_11); lean_dec(x_10); -lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -33212,33 +32469,39 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_32 = !lean_is_exclusive(x_18); -if (x_32 == 0) +x_41 = !lean_is_exclusive(x_35); +if (x_41 == 0) { -return x_18; +return x_35; } else { -lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_33 = lean_ctor_get(x_18, 0); -x_34 = lean_ctor_get(x_18, 1); -lean_inc(x_34); -lean_inc(x_33); -lean_dec(x_18); -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_42; lean_object* x_43; lean_object* x_44; +x_42 = lean_ctor_get(x_35, 0); +x_43 = lean_ctor_get(x_35, 1); +lean_inc(x_43); +lean_inc(x_42); +lean_dec(x_35); +x_44 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_44, 0, x_42); +lean_ctor_set(x_44, 1, x_43); +return x_44; } } } else { -uint8_t x_36; -lean_dec(x_12); +uint8_t x_45; +lean_dec(x_30); +lean_dec(x_18); +lean_dec(x_19); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); lean_dec(x_11); lean_dec(x_10); -lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -33247,187 +32510,39 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_36 = !lean_is_exclusive(x_16); -if (x_36 == 0) -{ -return x_16; -} -else -{ -lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_37 = lean_ctor_get(x_16, 0); -x_38 = lean_ctor_get(x_16, 1); -lean_inc(x_38); -lean_inc(x_37); -lean_dec(x_16); -x_39 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_39, 0, x_37); -lean_ctor_set(x_39, 1, x_38); -return x_39; -} -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { -_start: -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; -lean_inc(x_4); -x_14 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__5), 13, 5); -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_6); -x_15 = lean_unsigned_to_nat(0u); -x_16 = l_Lean_NameSet_empty; -x_17 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg(x_4, x_14, x_15, x_16, x_5, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -return x_17; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___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) { -_start: -{ -lean_object* x_12; lean_object* x_13; uint8_t x_14; -x_12 = lean_ctor_get(x_1, 0); -lean_inc(x_12); -lean_inc(x_12); -lean_inc(x_1); -x_13 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__6), 13, 4); -lean_closure_set(x_13, 0, x_2); -lean_closure_set(x_13, 1, x_1); -lean_closure_set(x_13, 2, x_12); -lean_closure_set(x_13, 3, x_3); -x_14 = !lean_is_exclusive(x_9); -if (x_14 == 0) +x_45 = !lean_is_exclusive(x_32); +if (x_45 == 0) { -lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = lean_ctor_get(x_9, 5); -x_16 = l_Lean_replaceRef(x_12, x_15); -lean_dec(x_15); -lean_dec(x_12); -lean_ctor_set(x_9, 5, x_16); -x_17 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents___rarg(x_1, x_13, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -return x_17; +return x_32; } 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; uint8_t x_29; lean_object* x_30; uint8_t x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_18 = lean_ctor_get(x_9, 0); -x_19 = lean_ctor_get(x_9, 1); -x_20 = lean_ctor_get(x_9, 2); -x_21 = lean_ctor_get(x_9, 3); -x_22 = lean_ctor_get(x_9, 4); -x_23 = lean_ctor_get(x_9, 5); -x_24 = lean_ctor_get(x_9, 6); -x_25 = lean_ctor_get(x_9, 7); -x_26 = lean_ctor_get(x_9, 8); -x_27 = lean_ctor_get(x_9, 9); -x_28 = lean_ctor_get(x_9, 10); -x_29 = lean_ctor_get_uint8(x_9, sizeof(void*)*12); -x_30 = lean_ctor_get(x_9, 11); -x_31 = lean_ctor_get_uint8(x_9, sizeof(void*)*12 + 1); -lean_inc(x_30); -lean_inc(x_28); -lean_inc(x_27); -lean_inc(x_26); -lean_inc(x_25); -lean_inc(x_24); -lean_inc(x_23); -lean_inc(x_22); -lean_inc(x_21); -lean_inc(x_20); -lean_inc(x_19); -lean_inc(x_18); -lean_dec(x_9); -x_32 = l_Lean_replaceRef(x_12, x_23); -lean_dec(x_23); -lean_dec(x_12); -x_33 = lean_alloc_ctor(0, 12, 2); -lean_ctor_set(x_33, 0, x_18); -lean_ctor_set(x_33, 1, x_19); -lean_ctor_set(x_33, 2, x_20); -lean_ctor_set(x_33, 3, x_21); -lean_ctor_set(x_33, 4, x_22); -lean_ctor_set(x_33, 5, x_32); -lean_ctor_set(x_33, 6, x_24); -lean_ctor_set(x_33, 7, x_25); -lean_ctor_set(x_33, 8, x_26); -lean_ctor_set(x_33, 9, x_27); -lean_ctor_set(x_33, 10, x_28); -lean_ctor_set(x_33, 11, x_30); -lean_ctor_set_uint8(x_33, sizeof(void*)*12, x_29); -lean_ctor_set_uint8(x_33, sizeof(void*)*12 + 1, x_31); -x_34 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents___rarg(x_1, x_13, x_5, x_6, x_7, x_8, x_33, x_10, x_11); -return x_34; -} -} -} -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("expected Type", 13, 13); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView(lean_object* x_1, lean_object* x_2, lean_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_29; lean_object* x_30; uint8_t x_31; -x_9 = lean_ctor_get(x_1, 10); -lean_inc(x_9); -x_29 = lean_array_get_size(x_9); -x_30 = lean_unsigned_to_nat(0u); -x_31 = lean_nat_dec_lt(x_30, x_29); -if (x_31 == 0) -{ -lean_dec(x_29); -x_10 = x_8; -goto block_28; +lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_46 = lean_ctor_get(x_32, 0); +x_47 = lean_ctor_get(x_32, 1); +lean_inc(x_47); +lean_inc(x_46); +lean_dec(x_32); +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_32; -x_32 = lean_nat_dec_le(x_29, x_29); -if (x_32 == 0) -{ -lean_dec(x_29); -x_10 = x_8; -goto block_28; } -else -{ -size_t x_33; size_t x_34; lean_object* x_35; lean_object* x_36; -x_33 = 0; -x_34 = lean_usize_of_nat(x_29); -lean_dec(x_29); -x_35 = lean_box(0); -lean_inc(x_6); -lean_inc(x_2); -x_36 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__11(x_1, x_9, x_33, x_34, x_35, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_36) == 0) -{ -lean_object* x_37; -x_37 = lean_ctor_get(x_36, 1); -lean_inc(x_37); -lean_dec(x_36); -x_10 = x_37; -goto block_28; } else { -uint8_t x_38; -lean_dec(x_9); +uint8_t x_49; +lean_dec(x_18); +lean_dec(x_19); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -33435,95 +32550,158 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_38 = !lean_is_exclusive(x_36); -if (x_38 == 0) +x_49 = !lean_is_exclusive(x_26); +if (x_49 == 0) { -return x_36; +return x_26; } else { -lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_39 = lean_ctor_get(x_36, 0); -x_40 = lean_ctor_get(x_36, 1); -lean_inc(x_40); -lean_inc(x_39); -lean_dec(x_36); -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_50; lean_object* x_51; lean_object* x_52; +x_50 = lean_ctor_get(x_26, 0); +x_51 = lean_ctor_get(x_26, 1); +lean_inc(x_51); +lean_inc(x_50); +lean_dec(x_26); +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; } } } -block_28: +else { -lean_object* x_11; lean_object* x_12; -x_11 = lean_ctor_get(x_1, 8); -lean_inc(x_11); -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_12 = l_Lean_Elab_Term_elabType(x_11, x_2, x_3, x_4, x_5, x_6, x_7, x_10); -if (lean_obj_tag(x_12) == 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; lean_object* x_62; lean_object* x_63; uint8_t x_64; lean_object* x_65; uint8_t x_66; lean_object* x_67; lean_object* x_68; uint8_t x_69; uint8_t x_70; lean_object* x_71; +x_53 = lean_ctor_get(x_18, 0); +x_54 = lean_ctor_get(x_18, 1); +x_55 = lean_ctor_get(x_18, 2); +x_56 = lean_ctor_get(x_18, 3); +x_57 = lean_ctor_get(x_18, 4); +x_58 = lean_ctor_get(x_18, 5); +x_59 = lean_ctor_get(x_18, 6); +x_60 = lean_ctor_get(x_18, 7); +x_61 = lean_ctor_get(x_18, 8); +x_62 = lean_ctor_get(x_18, 9); +x_63 = lean_ctor_get(x_18, 10); +x_64 = lean_ctor_get_uint8(x_18, sizeof(void*)*12); +x_65 = lean_ctor_get(x_18, 11); +x_66 = lean_ctor_get_uint8(x_18, sizeof(void*)*12 + 1); +lean_inc(x_65); +lean_inc(x_63); +lean_inc(x_62); +lean_inc(x_61); +lean_inc(x_60); +lean_inc(x_59); +lean_inc(x_58); +lean_inc(x_57); +lean_inc(x_56); +lean_inc(x_55); +lean_inc(x_54); +lean_inc(x_53); +lean_dec(x_18); +x_67 = l_Lean_replaceRef(x_1, x_58); +lean_dec(x_58); +x_68 = lean_alloc_ctor(0, 12, 2); +lean_ctor_set(x_68, 0, x_53); +lean_ctor_set(x_68, 1, x_54); +lean_ctor_set(x_68, 2, x_55); +lean_ctor_set(x_68, 3, x_56); +lean_ctor_set(x_68, 4, x_57); +lean_ctor_set(x_68, 5, x_67); +lean_ctor_set(x_68, 6, x_59); +lean_ctor_set(x_68, 7, x_60); +lean_ctor_set(x_68, 8, x_61); +lean_ctor_set(x_68, 9, x_62); +lean_ctor_set(x_68, 10, x_63); +lean_ctor_set(x_68, 11, x_65); +lean_ctor_set_uint8(x_68, sizeof(void*)*12, x_64); +lean_ctor_set_uint8(x_68, sizeof(void*)*12 + 1, x_66); +x_69 = 1; +x_70 = 0; +lean_inc(x_19); +lean_inc(x_68); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +x_71 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_69, x_70, x_14, x_15, x_16, x_17, x_68, x_19, x_20); +if (lean_obj_tag(x_71) == 0) { -lean_object* x_13; lean_object* x_14; uint8_t 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_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, 1); +lean_inc(x_72); +lean_dec(x_71); +x_73 = lean_ctor_get(x_2, 5); +lean_inc(x_73); +x_74 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_73, x_14, x_15, x_16, x_17, x_68, x_19, x_72); +x_75 = lean_ctor_get(x_74, 0); +lean_inc(x_75); +x_76 = lean_ctor_get(x_74, 1); +lean_inc(x_76); +lean_dec(x_74); +lean_inc(x_19); +lean_inc(x_68); +lean_inc(x_17); +lean_inc(x_16); lean_inc(x_14); -lean_dec(x_12); -x_15 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_validStructType(x_13); -if (x_15 == 0) +lean_inc(x_75); +x_77 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getResultUniverse(x_75, x_14, x_15, x_16, x_17, x_68, x_19, x_76); +if (lean_obj_tag(x_77) == 0) { -lean_object* x_16; lean_object* x_17; uint8_t x_18; +lean_object* x_78; lean_object* x_79; lean_object* x_80; +x_78 = lean_ctor_get(x_77, 0); +lean_inc(x_78); +x_79 = lean_ctor_get(x_77, 1); +lean_inc(x_79); +lean_dec(x_77); +lean_inc(x_14); +x_80 = l_Lean_Elab_Command_shouldInferResultUniverse(x_78, x_14, x_15, x_16, x_17, x_68, x_19, x_79); +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; +x_81 = lean_ctor_get(x_80, 0); +lean_inc(x_81); +x_82 = lean_ctor_get(x_80, 1); +lean_inc(x_82); +lean_dec(x_80); +x_83 = lean_box(x_9); +lean_inc(x_13); +lean_inc(x_3); +x_84 = lean_alloc_closure((void*)(l_Lean_Elab_Command_mkStructureDecl___lambda__5___boxed), 22, 14); +lean_closure_set(x_84, 0, x_3); +lean_closure_set(x_84, 1, x_13); +lean_closure_set(x_84, 2, x_81); +lean_closure_set(x_84, 3, x_4); +lean_closure_set(x_84, 4, x_2); +lean_closure_set(x_84, 5, x_5); +lean_closure_set(x_84, 6, x_6); +lean_closure_set(x_84, 7, x_7); +lean_closure_set(x_84, 8, x_8); +lean_closure_set(x_84, 9, x_83); +lean_closure_set(x_84, 10, x_1); +lean_closure_set(x_84, 11, x_10); +lean_closure_set(x_84, 12, x_11); +lean_closure_set(x_84, 13, x_75); +x_85 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withUsed___rarg(x_12, x_3, x_13, x_84, x_14, x_15, x_16, x_17, x_68, x_19, x_82); lean_dec(x_13); -lean_dec(x_9); -lean_dec(x_1); -x_16 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___closed__2; -x_17 = l_Lean_throwErrorAt___at___private_Lean_Elab_Binders_0__Lean_Elab_Term_elabBinderViews_loop___spec__1(x_11, x_16, x_2, x_3, x_4, x_5, x_6, x_7, x_14); -lean_dec(x_7); -lean_dec(x_5); -lean_dec(x_4); lean_dec(x_3); -lean_dec(x_11); -x_18 = !lean_is_exclusive(x_17); -if (x_18 == 0) -{ -return x_17; +return x_85; } 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_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; +lean_dec(x_75); +lean_dec(x_68); +lean_dec(x_19); lean_dec(x_17); -x_21 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_21, 0, x_19); -lean_ctor_set(x_21, 1, x_20); -return x_21; -} -} -else -{ -lean_object* x_22; lean_object* x_23; -lean_dec(x_11); -x_22 = lean_box(0); -x_23 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__7(x_1, x_13, x_9, x_22, x_2, x_3, x_4, x_5, x_6, x_7, x_14); -return x_23; -} -} -else -{ -uint8_t x_24; +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); lean_dec(x_11); -lean_dec(x_9); +lean_dec(x_10); +lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -33531,1832 +32709,1780 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_24 = !lean_is_exclusive(x_12); -if (x_24 == 0) -{ -return x_12; -} -else -{ -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_12, 0); -x_26 = lean_ctor_get(x_12, 1); -lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_12); -x_27 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_26); -return x_27; -} -} -} -} -} -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___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: -{ -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_Elab_Structure_0__Lean_Elab_Command_elabStructureView___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_1); -return x_14; +x_86 = lean_ctor_get(x_80, 0); +lean_inc(x_86); +x_87 = lean_ctor_get(x_80, 1); +lean_inc(x_87); +if (lean_is_exclusive(x_80)) { + lean_ctor_release(x_80, 0); + lean_ctor_release(x_80, 1); + x_88 = x_80; +} else { + lean_dec_ref(x_80); + x_88 = lean_box(0); } +if (lean_is_scalar(x_88)) { + x_89 = lean_alloc_ctor(1, 2, 0); +} else { + x_89 = x_88; } -LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___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_List_forM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_3); -lean_dec(x_2); -return x_9; +lean_ctor_set(x_89, 0, x_86); +lean_ctor_set(x_89, 1, x_87); +return x_89; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___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: +else { -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_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__4(x_11, x_12, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; +lean_dec(x_75); +lean_dec(x_68); +lean_dec(x_19); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_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); -return x_13; -} -} -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___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___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___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___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___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___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__6(x_1, x_5, x_6, x_4); -lean_dec(x_1); -return x_7; -} -} -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -size_t x_5; size_t x_6; lean_object* x_7; -x_5 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_6 = lean_unbox_usize(x_3); lean_dec(x_3); -x_7 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__7(x_1, x_5, x_6, x_4); -lean_dec(x_1); -return x_7; -} -} -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___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) { -_start: -{ -size_t x_15; size_t x_16; lean_object* x_17; -x_15 = lean_unbox_usize(x_5); -lean_dec(x_5); -x_16 = lean_unbox_usize(x_6); -lean_dec(x_6); -x_17 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__8(x_1, x_2, x_3, x_4, x_15, x_16, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_4); -return x_17; -} -} -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___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) { -_start: -{ -size_t x_12; size_t x_13; lean_object* x_14; -x_12 = lean_unbox_usize(x_2); lean_dec(x_2); -x_13 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_14 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__9(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; +x_90 = lean_ctor_get(x_77, 0); +lean_inc(x_90); +x_91 = lean_ctor_get(x_77, 1); +lean_inc(x_91); +if (lean_is_exclusive(x_77)) { + lean_ctor_release(x_77, 0); + lean_ctor_release(x_77, 1); + x_92 = x_77; +} else { + lean_dec_ref(x_77); + x_92 = lean_box(0); } +if (lean_is_scalar(x_92)) { + x_93 = lean_alloc_ctor(1, 2, 0); +} else { + x_93 = x_92; } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___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_2); -lean_dec(x_2); -x_6 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_7 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__10(x_1, x_5, x_6, x_4); -lean_dec(x_1); -return x_7; +lean_ctor_set(x_93, 0, x_90); +lean_ctor_set(x_93, 1, x_91); +return x_93; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__11___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +else { -lean_object* x_10; -x_10 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__11___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; +lean_dec(x_68); +lean_dec(x_19); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_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); -return x_10; +lean_dec(x_1); +x_94 = lean_ctor_get(x_71, 0); +lean_inc(x_94); +x_95 = lean_ctor_get(x_71, 1); +lean_inc(x_95); +if (lean_is_exclusive(x_71)) { + lean_ctor_release(x_71, 0); + lean_ctor_release(x_71, 1); + x_96 = x_71; +} else { + lean_dec_ref(x_71); + x_96 = lean_box(0); } +if (lean_is_scalar(x_96)) { + x_97 = lean_alloc_ctor(1, 2, 0); +} else { + x_97 = x_96; } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_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_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__11(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_2); -lean_dec(x_1); -return x_15; +lean_ctor_set(x_97, 0, x_94); +lean_ctor_set(x_97, 1, x_95); +return x_97; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; -x_10 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__1(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___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___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_Command_mkStructureDecl___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, uint8_t x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18) { _start: { -lean_object* x_12; -x_12 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_3); -lean_dec(x_2); -return x_12; -} +lean_object* x_19; lean_object* x_20; +x_19 = lean_ctor_get(x_1, 1); +lean_inc(x_19); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_2); +lean_inc(x_19); +x_20 = l_Lean_Elab_Term_addLocalVarInfo(x_19, x_2, x_12, x_13, x_14, x_15, x_16, x_17, x_18); +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; +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +x_22 = lean_ctor_get(x_1, 10); +lean_inc(x_22); +x_23 = lean_ctor_get(x_3, 7); +lean_inc(x_23); +x_24 = lean_box(x_8); +lean_inc(x_22); +x_25 = lean_alloc_closure((void*)(l_Lean_Elab_Command_mkStructureDecl___lambda__6___boxed), 20, 12); +lean_closure_set(x_25, 0, x_4); +lean_closure_set(x_25, 1, x_3); +lean_closure_set(x_25, 2, x_5); +lean_closure_set(x_25, 3, x_6); +lean_closure_set(x_25, 4, x_7); +lean_closure_set(x_25, 5, x_19); +lean_closure_set(x_25, 6, x_1); +lean_closure_set(x_25, 7, x_2); +lean_closure_set(x_25, 8, x_24); +lean_closure_set(x_25, 9, x_22); +lean_closure_set(x_25, 10, x_9); +lean_closure_set(x_25, 11, x_10); +x_26 = lean_unsigned_to_nat(0u); +x_27 = l_Lean_NameSet_empty; +x_28 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg(x_22, x_25, x_26, x_27, x_23, x_12, x_13, x_14, x_15, x_16, x_17, x_21); +return x_28; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___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 { -lean_object* x_17; -x_17 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +uint8_t x_29; +lean_dec(x_19); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_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_17; -} +lean_dec(x_2); +lean_dec(x_1); +x_29 = !lean_is_exclusive(x_20); +if (x_29 == 0) +{ +return x_20; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: +else { -lean_object* x_17; -x_17 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_7); -lean_dec(x_1); -return x_17; +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_20, 0); +x_31 = lean_ctor_get(x_20, 1); +lean_inc(x_31); +lean_inc(x_30); +lean_dec(x_20); +x_32 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_31); +return x_32; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -lean_object* x_12; -x_12 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__7(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; } } -static lean_object* _init_l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1___lambda__1___closed__1() { +static lean_object* _init_l_Lean_Elab_Command_mkStructureDecl___lambda__8___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("invalid use of 'partial' in inductive declaration", 49, 49); +x_1 = lean_mk_string_unchecked("indFVar: ", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1___lambda__1___closed__2() { +static lean_object* _init_l_Lean_Elab_Command_mkStructureDecl___lambda__8___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1___lambda__1___closed__1; +x_1 = l_Lean_Elab_Command_mkStructureDecl___lambda__8___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___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_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___lambda__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { -uint8_t x_6; -x_6 = l_Lean_Elab_Modifiers_isPartial(x_1); -if (x_6 == 0) +lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; +x_17 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__1; +x_18 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_17, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +x_20 = lean_unbox(x_19); +lean_dec(x_19); +if (x_20 == 0) { -lean_object* x_7; lean_object* x_8; -lean_dec(x_3); -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_5); -return x_8; +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_Lean_Elab_Command_mkStructureDecl___lambda__7(x_1, x_9, x_2, x_3, x_8, x_17, x_4, x_5, x_6, x_7, x_22, x_10, x_11, x_12, x_13, x_14, x_15, x_21); +return x_23; } else { -lean_object* x_9; lean_object* x_10; -x_9 = l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1___lambda__1___closed__2; -x_10 = l_Lean_throwError___at___private_Lean_Elab_Command_0__Lean_Elab_Command_elabCommandUsing___spec__1(x_9, x_3, x_4, x_5); -return x_10; +uint8_t x_24; +x_24 = !lean_is_exclusive(x_18); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_25 = lean_ctor_get(x_18, 1); +x_26 = lean_ctor_get(x_18, 0); +lean_dec(x_26); +lean_inc(x_9); +x_27 = l_Lean_MessageData_ofExpr(x_9); +x_28 = l_Lean_Elab_Command_mkStructureDecl___lambda__8___closed__2; +lean_ctor_set_tag(x_18, 7); +lean_ctor_set(x_18, 1, x_27); +lean_ctor_set(x_18, 0, x_28); +x_29 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3; +x_30 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_30, 0, x_18); +lean_ctor_set(x_30, 1, x_29); +x_31 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_17, x_30, x_10, x_11, x_12, x_13, x_14, x_15, x_25); +x_32 = lean_ctor_get(x_31, 0); +lean_inc(x_32); +x_33 = lean_ctor_get(x_31, 1); +lean_inc(x_33); +lean_dec(x_31); +x_34 = l_Lean_Elab_Command_mkStructureDecl___lambda__7(x_1, x_9, x_2, x_3, x_8, x_17, x_4, x_5, x_6, x_7, x_32, x_10, x_11, x_12, x_13, x_14, x_15, x_33); +lean_dec(x_32); +return x_34; } +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_35 = lean_ctor_get(x_18, 1); +lean_inc(x_35); +lean_dec(x_18); +lean_inc(x_9); +x_36 = l_Lean_MessageData_ofExpr(x_9); +x_37 = l_Lean_Elab_Command_mkStructureDecl___lambda__8___closed__2; +x_38 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_38, 0, x_37); +lean_ctor_set(x_38, 1, x_36); +x_39 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3; +x_40 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +x_41 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_17, x_40, x_10, x_11, x_12, x_13, x_14, x_15, x_35); +x_42 = lean_ctor_get(x_41, 0); +lean_inc(x_42); +x_43 = lean_ctor_get(x_41, 1); +lean_inc(x_43); +lean_dec(x_41); +x_44 = l_Lean_Elab_Command_mkStructureDecl___lambda__7(x_1, x_9, x_2, x_3, x_8, x_17, x_4, x_5, x_6, x_7, x_42, x_10, x_11, x_12, x_13, x_14, x_15, x_43); +lean_dec(x_42); +return x_44; } } -static lean_object* _init_l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("invalid use of 'noncomputable' in inductive declaration", 55, 55); -return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1___closed__2() { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___lambda__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} +lean_object* x_14; +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_1); +x_14 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader(x_1, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_14) == 0) +{ +lean_object* x_15; lean_object* x_16; uint8_t x_17; uint8_t x_18; lean_object* x_19; +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); +x_17 = 1; +x_18 = 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_19 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_17, x_18, x_7, x_8, x_9, x_10, x_11, x_12, x_16); +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; +x_20 = lean_ctor_get(x_19, 1); +lean_inc(x_20); +lean_dec(x_19); +x_21 = lean_ctor_get(x_15, 1); +lean_inc(x_21); +x_22 = lean_ctor_get(x_15, 2); +lean_inc(x_22); +x_23 = lean_box(x_4); +lean_inc(x_15); +x_24 = lean_alloc_closure((void*)(l_Lean_Elab_Command_mkStructureDecl___lambda__8___boxed), 16, 7); +lean_closure_set(x_24, 0, x_1); +lean_closure_set(x_24, 1, x_15); +lean_closure_set(x_24, 2, x_2); +lean_closure_set(x_24, 3, x_3); +lean_closure_set(x_24, 4, x_23); +lean_closure_set(x_24, 5, x_5); +lean_closure_set(x_24, 6, x_6); +x_25 = lean_alloc_closure((void*)(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withStructureLocalDecl___rarg), 9, 2); +lean_closure_set(x_25, 0, x_15); +lean_closure_set(x_25, 1, x_24); +x_26 = l_Lean_Meta_withLCtx___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__3___rarg(x_21, x_22, x_25, x_7, x_8, x_9, x_10, x_11, x_12, x_20); +return x_26; } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: +else { -uint8_t x_5; -x_5 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 1); -if (x_5 == 0) +uint8_t x_27; +lean_dec(x_15); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_27 = !lean_is_exclusive(x_19); +if (x_27 == 0) { -lean_object* x_6; lean_object* x_7; -x_6 = lean_box(0); -x_7 = l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1___lambda__1(x_1, x_6, x_2, x_3, x_4); -return x_7; +return x_19; } else { -lean_object* x_8; lean_object* x_9; uint8_t x_10; -x_8 = l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1___closed__2; -x_9 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_8, x_2, x_3, x_4); -x_10 = !lean_is_exclusive(x_9); -if (x_10 == 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 { -return x_9; +uint8_t x_31; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_31 = !lean_is_exclusive(x_14); +if (x_31 == 0) +{ +return x_14; } else { -lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_11 = lean_ctor_get(x_9, 0); -x_12 = lean_ctor_get(x_9, 1); -lean_inc(x_12); +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_14, 0); +x_33 = lean_ctor_get(x_14, 1); +lean_inc(x_33); +lean_inc(x_32); +lean_dec(x_14); +x_34 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_34, 0, x_32); +lean_ctor_set(x_34, 1, x_33); +return x_34; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___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) { +_start: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; +x_10 = l_Lean_Elab_Term_getLevelNames___rarg(x_4, x_5, x_6, x_7, x_8, x_9); +x_11 = lean_ctor_get(x_10, 0); lean_inc(x_11); -lean_dec(x_9); -x_13 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_13, 0, x_11); -lean_ctor_set(x_13, 1, x_12); -return x_13; +x_12 = lean_ctor_get(x_10, 1); +lean_inc(x_12); +lean_dec(x_10); +x_13 = lean_ctor_get(x_1, 2); +lean_inc(x_13); +x_14 = lean_ctor_get_uint8(x_13, sizeof(void*)*3 + 3); +x_15 = lean_ctor_get(x_1, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_1, 5); +lean_inc(x_16); +x_17 = lean_box(x_14); +lean_inc(x_15); +x_18 = lean_alloc_closure((void*)(l_Lean_Elab_Command_mkStructureDecl___lambda__9___boxed), 13, 6); +lean_closure_set(x_18, 0, x_1); +lean_closure_set(x_18, 1, x_15); +lean_closure_set(x_18, 2, x_11); +lean_closure_set(x_18, 3, x_17); +lean_closure_set(x_18, 4, x_13); +lean_closure_set(x_18, 5, x_2); +x_19 = !lean_is_exclusive(x_7); +if (x_19 == 0) +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_7, 5); +x_21 = l_Lean_replaceRef(x_15, x_20); +lean_dec(x_20); +lean_dec(x_15); +lean_ctor_set(x_7, 5, x_21); +x_22 = l_Lean_Elab_Term_withLevelNames___rarg(x_16, x_18, x_3, x_4, x_5, x_6, x_7, x_8, x_12); +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_33; uint8_t x_34; lean_object* x_35; uint8_t x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_23 = lean_ctor_get(x_7, 0); +x_24 = lean_ctor_get(x_7, 1); +x_25 = lean_ctor_get(x_7, 2); +x_26 = lean_ctor_get(x_7, 3); +x_27 = lean_ctor_get(x_7, 4); +x_28 = lean_ctor_get(x_7, 5); +x_29 = lean_ctor_get(x_7, 6); +x_30 = lean_ctor_get(x_7, 7); +x_31 = lean_ctor_get(x_7, 8); +x_32 = lean_ctor_get(x_7, 9); +x_33 = lean_ctor_get(x_7, 10); +x_34 = lean_ctor_get_uint8(x_7, sizeof(void*)*12); +x_35 = lean_ctor_get(x_7, 11); +x_36 = lean_ctor_get_uint8(x_7, sizeof(void*)*12 + 1); +lean_inc(x_35); +lean_inc(x_33); +lean_inc(x_32); +lean_inc(x_31); +lean_inc(x_30); +lean_inc(x_29); +lean_inc(x_28); +lean_inc(x_27); +lean_inc(x_26); +lean_inc(x_25); +lean_inc(x_24); +lean_inc(x_23); +lean_dec(x_7); +x_37 = l_Lean_replaceRef(x_15, x_28); +lean_dec(x_28); +lean_dec(x_15); +x_38 = lean_alloc_ctor(0, 12, 2); +lean_ctor_set(x_38, 0, x_23); +lean_ctor_set(x_38, 1, x_24); +lean_ctor_set(x_38, 2, x_25); +lean_ctor_set(x_38, 3, x_26); +lean_ctor_set(x_38, 4, x_27); +lean_ctor_set(x_38, 5, x_37); +lean_ctor_set(x_38, 6, x_29); +lean_ctor_set(x_38, 7, x_30); +lean_ctor_set(x_38, 8, x_31); +lean_ctor_set(x_38, 9, x_32); +lean_ctor_set(x_38, 10, x_33); +lean_ctor_set(x_38, 11, x_35); +lean_ctor_set_uint8(x_38, sizeof(void*)*12, x_34); +lean_ctor_set_uint8(x_38, sizeof(void*)*12 + 1, x_36); +x_39 = l_Lean_Elab_Term_withLevelNames___rarg(x_16, x_18, x_3, x_4, x_5, x_6, x_38, x_8, x_12); +return x_39; } } } -static lean_object* _init_l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___spec__2___closed__1() { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("example", 7, 7); -return x_1; +lean_object* x_10; lean_object* x_11; +x_10 = lean_alloc_closure((void*)(l_Lean_Elab_Command_mkStructureDecl___lambda__10), 9, 2); +lean_closure_set(x_10, 0, x_2); +lean_closure_set(x_10, 1, x_1); +x_11 = l_Lean_Elab_Term_withoutSavingRecAppSyntax___rarg(x_10, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_11; } } -static lean_object* _init_l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___spec__2___closed__2() { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_mkStructureDecl___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_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__1; -x_2 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__2; -x_3 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__1; -x_4 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___spec__2___closed__1; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; +size_t x_12; size_t x_13; lean_object* x_14; +x_12 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_13 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_14 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_mkStructureDecl___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; } } -LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_List_forM___at_Lean_Elab_Command_mkStructureDecl___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) { _start: { -lean_object* x_10; lean_object* x_11; uint8_t x_12; -lean_inc(x_2); -x_10 = l_Lean_Syntax_getKind(x_2); -x_11 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___spec__2___closed__2; -x_12 = lean_name_eq(x_10, x_11); -lean_dec(x_10); -if (x_12 == 0) -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; -lean_inc(x_7); -x_13 = l_Lean_Elab_getDeclarationRange___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__19(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -x_14 = lean_ctor_get(x_13, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_13, 1); -lean_inc(x_15); -lean_dec(x_13); -x_16 = l_Lean_Elab_getDeclarationSelectionRef(x_2); -lean_inc(x_7); -x_17 = l_Lean_Elab_getDeclarationRange___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__19(x_16, x_3, x_4, x_5, x_6, x_7, x_8, x_15); -lean_dec(x_16); -x_18 = !lean_is_exclusive(x_17); -if (x_18 == 0) -{ -lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_19 = lean_ctor_get(x_17, 0); -x_20 = lean_ctor_get(x_17, 1); -lean_ctor_set(x_17, 1, x_19); -lean_ctor_set(x_17, 0, x_14); -x_21 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20(x_1, x_17, x_3, x_4, x_5, x_6, x_7, x_8, x_20); -lean_dec(x_7); -return x_21; +lean_object* x_9; +x_9 = l_List_forM___at_Lean_Elab_Command_mkStructureDecl___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_3); +lean_dec(x_2); +return x_9; } -else +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_mkStructureDecl___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: { -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_22 = lean_ctor_get(x_17, 0); -x_23 = lean_ctor_get(x_17, 1); -lean_inc(x_23); -lean_inc(x_22); -lean_dec(x_17); -x_24 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_24, 0, x_14); -lean_ctor_set(x_24, 1, x_22); -x_25 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20(x_1, x_24, x_3, x_4, x_5, x_6, x_7, x_8, x_23); -lean_dec(x_7); -return x_25; +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_Command_mkStructureDecl___spec__3(x_1, x_5, x_6, x_4); +lean_dec(x_1); +return x_7; } } -else +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_mkStructureDecl___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: { -lean_object* x_26; lean_object* x_27; -lean_dec(x_7); +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_Command_mkStructureDecl___spec__4(x_1, x_5, x_6, x_4); lean_dec(x_1); -x_26 = lean_box(0); -x_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_26); -lean_ctor_set(x_27, 1, x_9); -return x_27; -} +return x_7; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabStructure___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_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_mkStructureDecl___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { -uint8_t x_9; -x_9 = lean_usize_dec_eq(x_3, x_4); -if (x_9 == 0) -{ -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +size_t x_15; size_t x_16; lean_object* x_17; +x_15 = lean_unbox_usize(x_5); lean_dec(x_5); -x_10 = lean_array_uget(x_2, x_3); -x_11 = lean_box(0); -lean_inc(x_1); -x_12 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_12, 0, x_1); -lean_ctor_set(x_12, 1, x_11); -x_13 = lean_array_mk(x_12); -lean_inc(x_7); -lean_inc(x_6); -x_14 = l_Lean_Elab_DerivingClassView_applyHandlers(x_10, x_13, x_6, x_7, x_8); -if (lean_obj_tag(x_14) == 0) -{ -lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; -x_15 = lean_ctor_get(x_14, 0); -lean_inc(x_15); -x_16 = lean_ctor_get(x_14, 1); -lean_inc(x_16); -lean_dec(x_14); -x_17 = 1; -x_18 = lean_usize_add(x_3, x_17); -x_3 = x_18; -x_5 = x_15; -x_8 = x_16; -goto _start; -} -else -{ -uint8_t x_20; -lean_dec(x_7); +x_16 = lean_unbox_usize(x_6); lean_dec(x_6); -lean_dec(x_1); -x_20 = !lean_is_exclusive(x_14); -if (x_20 == 0) -{ -return x_14; -} -else -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_14, 0); -x_22 = lean_ctor_get(x_14, 1); -lean_inc(x_22); -lean_inc(x_21); -lean_dec(x_14); -x_23 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_23, 0, x_21); -lean_ctor_set(x_23, 1, x_22); -return x_23; -} +x_17 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_mkStructureDecl___spec__5(x_1, x_2, x_3, x_4, x_15, x_16, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_4); +return x_17; } } -else +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_mkStructureDecl___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) { +_start: { -lean_object* x_24; -lean_dec(x_7); -lean_dec(x_6); +size_t x_12; size_t x_13; lean_object* x_14; +x_12 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_13 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_14 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_mkStructureDecl___spec__6(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); -x_24 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_24, 0, x_5); -lean_ctor_set(x_24, 1, x_8); -return x_24; -} +return x_14; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, 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_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_1); -lean_ctor_set(x_10, 1, x_9); +x_10 = l_Lean_Elab_Command_mkStructureDecl___lambda__1(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_Lean_Elab_Command_elabStructure___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, 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_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -uint8_t x_20; uint8_t x_21; lean_object* x_22; -x_20 = 1; -x_21 = 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); -x_22 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_20, x_21, x_13, x_14, x_15, x_16, x_17, x_18, x_19); -if (lean_obj_tag(x_22) == 0) -{ -lean_object* x_23; lean_object* x_24; -x_23 = lean_ctor_get(x_22, 1); -lean_inc(x_23); -lean_dec(x_22); -lean_inc(x_18); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_15); -lean_inc(x_13); -x_24 = l_Lean_Elab_Term_addAutoBoundImplicits(x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_23); -if (lean_obj_tag(x_24) == 0) -{ -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; -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_getLevelNames___rarg(x_14, x_15, x_16, x_17, x_18, 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); -lean_inc(x_5); -x_30 = lean_alloc_ctor(0, 11, 1); -lean_ctor_set(x_30, 0, x_1); -lean_ctor_set(x_30, 1, x_2); -lean_ctor_set(x_30, 2, x_3); -lean_ctor_set(x_30, 3, x_28); -lean_ctor_set(x_30, 4, x_5); -lean_ctor_set(x_30, 5, x_6); -lean_ctor_set(x_30, 6, x_25); -lean_ctor_set(x_30, 7, x_7); -lean_ctor_set(x_30, 8, x_8); -lean_ctor_set(x_30, 9, x_9); -lean_ctor_set(x_30, 10, x_10); -lean_ctor_set_uint8(x_30, sizeof(void*)*11, x_4); -lean_inc(x_18); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_15); -x_31 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView(x_30, x_13, x_14, x_15, x_16, x_17, x_18, x_29); -if (lean_obj_tag(x_31) == 0) -{ -if (x_11 == 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); -lean_inc(x_18); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_15); -lean_inc(x_5); -x_33 = l_Lean_Meta_mkSizeOfInstances(x_5, x_15, x_16, x_17, x_18, x_32); -if (lean_obj_tag(x_33) == 0) -{ -lean_object* x_34; lean_object* x_35; -x_34 = lean_ctor_get(x_33, 1); -lean_inc(x_34); -lean_dec(x_33); -lean_inc(x_5); -x_35 = l_Lean_Meta_mkInjectiveTheorems(x_5, x_15, x_16, x_17, x_18, x_34); -if (lean_obj_tag(x_35) == 0) -{ -uint8_t x_36; -x_36 = !lean_is_exclusive(x_35); -if (x_36 == 0) -{ -lean_object* x_37; -x_37 = lean_ctor_get(x_35, 0); -lean_dec(x_37); -lean_ctor_set(x_35, 0, x_5); -return x_35; -} -else -{ -lean_object* x_38; lean_object* x_39; -x_38 = lean_ctor_get(x_35, 1); -lean_inc(x_38); -lean_dec(x_35); -x_39 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_39, 0, x_5); -lean_ctor_set(x_39, 1, x_38); -return x_39; -} +lean_object* x_12; +x_12 = l_Lean_Elab_Command_mkStructureDecl___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_3); +lean_dec(x_2); +return x_12; } -else -{ -uint8_t x_40; -lean_dec(x_5); -x_40 = !lean_is_exclusive(x_35); -if (x_40 == 0) -{ -return x_35; } -else +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___lambda__3___boxed(lean_object** _args) { +lean_object* x_1 = _args[0]; +lean_object* x_2 = _args[1]; +lean_object* x_3 = _args[2]; +lean_object* x_4 = _args[3]; +lean_object* x_5 = _args[4]; +lean_object* x_6 = _args[5]; +lean_object* x_7 = _args[6]; +lean_object* x_8 = _args[7]; +lean_object* x_9 = _args[8]; +lean_object* x_10 = _args[9]; +lean_object* x_11 = _args[10]; +lean_object* x_12 = _args[11]; +lean_object* x_13 = _args[12]; +lean_object* x_14 = _args[13]; +lean_object* x_15 = _args[14]; +lean_object* x_16 = _args[15]; +lean_object* x_17 = _args[16]; +lean_object* x_18 = _args[17]; +_start: { -lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_ctor_get(x_35, 0); -x_42 = lean_ctor_get(x_35, 1); -lean_inc(x_42); -lean_inc(x_41); -lean_dec(x_35); -x_43 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_43, 0, x_41); -lean_ctor_set(x_43, 1, x_42); -return x_43; -} +lean_object* x_19; +x_19 = l_Lean_Elab_Command_mkStructureDecl___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18); +lean_dec(x_9); +lean_dec(x_8); +return x_19; } } -else -{ -uint8_t x_44; -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_5); -x_44 = !lean_is_exclusive(x_33); -if (x_44 == 0) +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___lambda__4___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]; +_start: { -return x_33; +uint8_t x_22; lean_object* x_23; +x_22 = lean_unbox(x_10); +lean_dec(x_10); +x_23 = l_Lean_Elab_Command_mkStructureDecl___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_22, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20, x_21); +lean_dec(x_14); +lean_dec(x_3); +return x_23; } -else -{ -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_33, 0); -x_46 = lean_ctor_get(x_33, 1); -lean_inc(x_46); -lean_inc(x_45); -lean_dec(x_33); -x_47 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_47, 0, x_45); -lean_ctor_set(x_47, 1, x_46); -return x_47; } +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___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]; +lean_object* x_18 = _args[17]; +lean_object* x_19 = _args[18]; +lean_object* x_20 = _args[19]; +lean_object* x_21 = _args[20]; +lean_object* x_22 = _args[21]; +_start: +{ +uint8_t x_23; lean_object* x_24; +x_23 = lean_unbox(x_10); +lean_dec(x_10); +x_24 = l_Lean_Elab_Command_mkStructureDecl___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_23, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20, x_21, x_22); +lean_dec(x_1); +return x_24; } } -else -{ -uint8_t x_48; -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -x_48 = !lean_is_exclusive(x_31); -if (x_48 == 0) +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___lambda__6___boxed(lean_object** _args) { +lean_object* x_1 = _args[0]; +lean_object* x_2 = _args[1]; +lean_object* x_3 = _args[2]; +lean_object* x_4 = _args[3]; +lean_object* x_5 = _args[4]; +lean_object* x_6 = _args[5]; +lean_object* x_7 = _args[6]; +lean_object* x_8 = _args[7]; +lean_object* x_9 = _args[8]; +lean_object* x_10 = _args[9]; +lean_object* x_11 = _args[10]; +lean_object* x_12 = _args[11]; +lean_object* x_13 = _args[12]; +lean_object* x_14 = _args[13]; +lean_object* x_15 = _args[14]; +lean_object* x_16 = _args[15]; +lean_object* x_17 = _args[16]; +lean_object* x_18 = _args[17]; +lean_object* x_19 = _args[18]; +lean_object* x_20 = _args[19]; +_start: { -lean_object* x_49; -x_49 = lean_ctor_get(x_31, 0); -lean_dec(x_49); -lean_ctor_set(x_31, 0, x_5); -return x_31; +uint8_t x_21; lean_object* x_22; +x_21 = lean_unbox(x_9); +lean_dec(x_9); +x_22 = l_Lean_Elab_Command_mkStructureDecl___lambda__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_21, 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_12); +return x_22; } -else -{ -lean_object* x_50; lean_object* x_51; -x_50 = lean_ctor_get(x_31, 1); -lean_inc(x_50); -lean_dec(x_31); -x_51 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_51, 0, x_5); -lean_ctor_set(x_51, 1, x_50); -return x_51; } +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___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]; +lean_object* x_18 = _args[17]; +_start: +{ +uint8_t x_19; lean_object* x_20; +x_19 = lean_unbox(x_8); +lean_dec(x_8); +x_20 = l_Lean_Elab_Command_mkStructureDecl___lambda__7(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_19, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18); +lean_dec(x_11); +return x_20; } } -else +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___lambda__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +_start: { -uint8_t x_52; -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); +uint8_t x_17; lean_object* x_18; +x_17 = lean_unbox(x_5); lean_dec(x_5); -x_52 = !lean_is_exclusive(x_31); -if (x_52 == 0) -{ -return x_31; +x_18 = l_Lean_Elab_Command_mkStructureDecl___lambda__8(x_1, x_2, x_3, x_4, x_17, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +return x_18; } -else -{ -lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_53 = lean_ctor_get(x_31, 0); -x_54 = lean_ctor_get(x_31, 1); -lean_inc(x_54); -lean_inc(x_53); -lean_dec(x_31); -x_55 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_55, 0, x_53); -lean_ctor_set(x_55, 1, x_54); -return x_55; } +LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkStructureDecl___lambda__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +uint8_t x_14; lean_object* x_15; +x_14 = lean_unbox(x_4); +lean_dec(x_4); +x_15 = l_Lean_Elab_Command_mkStructureDecl___lambda__9(x_1, x_2, x_3, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +return x_15; } } -else +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructureView___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_56; -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); +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_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); +lean_ctor_set(x_9, 5, x_14); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_3); +x_15 = l_Lean_Elab_Command_mkStructureDecl(x_2, x_3, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_15) == 0) +{ +uint8_t x_16; +x_16 = lean_ctor_get_uint8(x_3, sizeof(void*)*12); lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_56 = !lean_is_exclusive(x_24); -if (x_56 == 0) +if (x_16 == 0) { -return x_24; -} -else +lean_object* x_17; lean_object* x_18; +x_17 = lean_ctor_get(x_15, 1); +lean_inc(x_17); +lean_dec(x_15); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_4); +x_18 = l_Lean_Meta_IndPredBelow_mkBelow(x_4, x_7, x_8, x_9, x_10, x_17); +if (lean_obj_tag(x_18) == 0) { -lean_object* x_57; lean_object* x_58; lean_object* x_59; -x_57 = lean_ctor_get(x_24, 0); -x_58 = lean_ctor_get(x_24, 1); -lean_inc(x_58); -lean_inc(x_57); -lean_dec(x_24); -x_59 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_59, 0, x_57); -lean_ctor_set(x_59, 1, x_58); -return x_59; -} -} +lean_object* x_19; lean_object* x_20; +x_19 = lean_ctor_get(x_18, 1); +lean_inc(x_19); +lean_dec(x_18); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_4); +x_20 = l_Lean_Meta_mkSizeOfInstances(x_4, x_7, x_8, x_9, x_10, x_19); +if (lean_obj_tag(x_20) == 0) +{ +lean_object* x_21; lean_object* x_22; +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +x_22 = l_Lean_Meta_mkInjectiveTheorems(x_4, x_7, x_8, x_9, x_10, x_21); +return x_22; } else { -uint8_t x_60; -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_10); +uint8_t x_23; lean_dec(x_9); +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_2); -lean_dec(x_1); -x_60 = !lean_is_exclusive(x_22); -if (x_60 == 0) +lean_dec(x_4); +x_23 = !lean_is_exclusive(x_20); +if (x_23 == 0) { -return x_22; +return x_20; } else { -lean_object* x_61; lean_object* x_62; lean_object* x_63; -x_61 = lean_ctor_get(x_22, 0); -x_62 = lean_ctor_get(x_22, 1); -lean_inc(x_62); -lean_inc(x_61); -lean_dec(x_22); -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; -} -} +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_20, 0); +x_25 = lean_ctor_get(x_20, 1); +lean_inc(x_25); +lean_inc(x_24); +lean_dec(x_20); +x_26 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_26, 0, x_24); +lean_ctor_set(x_26, 1, x_25); +return x_26; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, uint8_t x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18) { -_start: -{ -lean_object* x_19; -lean_inc(x_16); -lean_inc(x_12); -lean_inc(x_3); -x_19 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor(x_1, x_2, x_3, x_12, x_13, x_14, x_15, x_16, x_17, x_18); -if (lean_obj_tag(x_19) == 0) -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_19, 1); -lean_inc(x_21); -lean_dec(x_19); -lean_inc(x_17); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_3); -x_22 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields(x_1, x_2, x_3, x_12, x_13, x_14, x_15, x_16, x_17, x_21); -if (lean_obj_tag(x_22) == 0) -{ -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -x_24 = lean_ctor_get(x_22, 1); -lean_inc(x_24); -lean_dec(x_22); -x_25 = lean_box(x_5); -x_26 = lean_box(x_9); -x_27 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabStructure___lambda__2___boxed), 19, 11); -lean_closure_set(x_27, 0, x_1); -lean_closure_set(x_27, 1, x_2); -lean_closure_set(x_27, 2, x_4); -lean_closure_set(x_27, 3, x_25); -lean_closure_set(x_27, 4, x_3); -lean_closure_set(x_27, 5, x_6); -lean_closure_set(x_27, 6, x_7); -lean_closure_set(x_27, 7, x_8); -lean_closure_set(x_27, 8, x_20); -lean_closure_set(x_27, 9, x_23); -lean_closure_set(x_27, 10, x_26); -x_28 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabBinders___rarg), 9, 2); -lean_closure_set(x_28, 0, x_10); -lean_closure_set(x_28, 1, x_27); -x_29 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withAutoBoundImplicit___rarg), 8, 1); -lean_closure_set(x_29, 0, x_28); -x_30 = l_Lean_Elab_Term_withLevelNames___rarg(x_11, x_29, x_12, x_13, x_14, x_15, x_16, x_17, x_24); -return x_30; } else { -uint8_t x_31; -lean_dec(x_20); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); +uint8_t x_27; +lean_dec(x_9); lean_dec(x_10); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_31 = !lean_is_exclusive(x_22); -if (x_31 == 0) +x_27 = !lean_is_exclusive(x_18); +if (x_27 == 0) { -return x_22; +return x_18; } else { -lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_32 = lean_ctor_get(x_22, 0); -x_33 = lean_ctor_get(x_22, 1); -lean_inc(x_33); -lean_inc(x_32); -lean_dec(x_22); -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_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_18, 0); +x_29 = lean_ctor_get(x_18, 1); +lean_inc(x_29); +lean_inc(x_28); +lean_dec(x_18); +x_30 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +return x_30; } } } else { -uint8_t x_35; -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); +uint8_t x_31; +lean_dec(x_9); lean_dec(x_10); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_35 = !lean_is_exclusive(x_19); -if (x_35 == 0) +x_31 = !lean_is_exclusive(x_15); +if (x_31 == 0) { -return x_19; +lean_object* x_32; lean_object* x_33; +x_32 = lean_ctor_get(x_15, 0); +lean_dec(x_32); +x_33 = lean_box(0); +lean_ctor_set(x_15, 0, x_33); +return x_15; } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_19, 0); -x_37 = lean_ctor_get(x_19, 1); -lean_inc(x_37); -lean_inc(x_36); -lean_dec(x_19); -x_38 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -return x_38; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, uint8_t x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18) { -_start: -{ -lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; -lean_inc(x_16); -lean_inc(x_2); -lean_inc(x_1); -x_19 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___spec__2(x_1, x_2, x_12, x_13, x_14, x_15, x_16, x_17, x_18); -x_20 = lean_ctor_get(x_19, 1); -lean_inc(x_20); -lean_dec(x_19); -x_21 = lean_box(x_5); -x_22 = lean_box(x_9); -lean_inc(x_1); -x_23 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabStructure___lambda__3___boxed), 18, 11); -lean_closure_set(x_23, 0, x_2); -lean_closure_set(x_23, 1, x_3); -lean_closure_set(x_23, 2, x_1); -lean_closure_set(x_23, 3, x_4); -lean_closure_set(x_23, 4, x_21); -lean_closure_set(x_23, 5, x_6); -lean_closure_set(x_23, 6, x_7); -lean_closure_set(x_23, 7, x_8); -lean_closure_set(x_23, 8, x_22); -lean_closure_set(x_23, 9, x_10); -lean_closure_set(x_23, 10, x_11); -x_24 = l_Lean_Elab_Term_withDeclName___rarg(x_1, x_23, x_12, x_13, x_14, x_15, x_16, x_17, x_20); -return x_24; +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_15, 1); +lean_inc(x_34); +lean_dec(x_15); +x_35 = lean_box(0); +x_36 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_36, 0, x_35); +lean_ctor_set(x_36, 1, x_34); +return x_36; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, uint8_t x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_17 = l_Lean_Elab_Term_getLevelNames___rarg(x_11, x_12, x_13, x_14, x_15, x_16); -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_17, 1); -lean_inc(x_19); -lean_dec(x_17); -x_20 = lean_ctor_get(x_14, 6); -lean_inc(x_20); -lean_inc(x_14); -lean_inc(x_10); -lean_inc(x_2); -lean_inc(x_18); -x_21 = l_Lean_Elab_expandDeclId___at_Lean_Elab_Term_expandDeclId___spec__1(x_20, x_18, x_1, x_2, x_10, x_11, x_12, x_13, x_14, x_15, x_19); -if (lean_obj_tag(x_21) == 0) -{ -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_22 = lean_ctor_get(x_21, 0); -lean_inc(x_22); -x_23 = lean_ctor_get(x_21, 1); -lean_inc(x_23); -lean_dec(x_21); -x_24 = lean_ctor_get(x_22, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_22, 1); -lean_inc(x_25); -x_26 = lean_ctor_get(x_22, 2); -lean_inc(x_26); -lean_dec(x_22); -x_27 = lean_alloc_closure((void*)(l_Lean_Name_beq___boxed), 2, 1); -lean_closure_set(x_27, 0, x_24); -x_28 = lean_box(x_4); -x_29 = lean_box(x_7); -x_30 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabStructure___lambda__4___boxed), 18, 11); -lean_closure_set(x_30, 0, x_25); -lean_closure_set(x_30, 1, x_3); -lean_closure_set(x_30, 2, x_2); -lean_closure_set(x_30, 3, x_18); -lean_closure_set(x_30, 4, x_28); -lean_closure_set(x_30, 5, x_9); -lean_closure_set(x_30, 6, x_5); -lean_closure_set(x_30, 7, x_6); -lean_closure_set(x_30, 8, x_29); -lean_closure_set(x_30, 9, x_8); -lean_closure_set(x_30, 10, x_26); -x_31 = l_Lean_Elab_Term_withAutoBoundImplicitForbiddenPred___rarg(x_27, x_30, x_10, x_11, x_12, x_13, x_14, x_15, x_23); -return x_31; } else { -uint8_t x_32; -lean_dec(x_18); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); +uint8_t x_37; lean_dec(x_9); +lean_dec(x_10); lean_dec(x_8); -lean_dec(x_6); -lean_dec(x_5); +lean_dec(x_7); +lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); -x_32 = !lean_is_exclusive(x_21); -if (x_32 == 0) +x_37 = !lean_is_exclusive(x_15); +if (x_37 == 0) { -return x_21; +return x_15; } else { -lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_33 = lean_ctor_get(x_21, 0); -x_34 = lean_ctor_get(x_21, 1); -lean_inc(x_34); -lean_inc(x_33); -lean_dec(x_21); -x_35 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_35, 0, x_33); -lean_ctor_set(x_35, 1, x_34); -return x_35; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; uint8_t x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_11 = lean_ctor_get(x_1, 1); -lean_inc(x_11); -lean_dec(x_1); -x_12 = 1; -x_13 = lean_box(x_12); -lean_inc(x_2); -x_14 = lean_alloc_closure((void*)(l_Lean_Elab_Term_applyAttributesAt___boxed), 10, 3); -lean_closure_set(x_14, 0, x_2); -lean_closure_set(x_14, 1, x_11); -lean_closure_set(x_14, 2, x_13); -x_15 = l_Lean_Elab_Term_withDeclName___rarg(x_2, x_14, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_15; +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_15, 0); +x_39 = lean_ctor_get(x_15, 1); +lean_inc(x_39); +lean_inc(x_38); +lean_dec(x_15); +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_Command_elabStructure___lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_13 = lean_box(x_4); -x_14 = lean_box(x_6); -lean_inc(x_2); -x_15 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabStructure___lambda__5___boxed), 16, 8); -lean_closure_set(x_15, 0, x_1); -lean_closure_set(x_15, 1, x_2); -lean_closure_set(x_15, 2, x_3); -lean_closure_set(x_15, 3, x_13); -lean_closure_set(x_15, 4, x_5); -lean_closure_set(x_15, 5, x_9); -lean_closure_set(x_15, 6, x_14); -lean_closure_set(x_15, 7, x_7); -x_16 = l_Lean_Elab_Command_runTermElabM___rarg(x_15, 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; uint8_t x_21; -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_16, 1); -lean_inc(x_18); -lean_dec(x_16); -x_19 = lean_array_get_size(x_8); -x_20 = lean_unsigned_to_nat(0u); -x_21 = lean_nat_dec_lt(x_20, x_19); -if (x_21 == 0) -{ -lean_object* x_22; lean_object* x_23; -lean_dec(x_19); -x_22 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabStructure___lambda__6___boxed), 10, 2); -lean_closure_set(x_22, 0, x_2); -lean_closure_set(x_22, 1, x_17); -x_23 = l_Lean_Elab_Command_runTermElabM___rarg(x_22, x_10, x_11, x_18); -lean_dec(x_11); -lean_dec(x_10); -return x_23; } else { -uint8_t x_24; -x_24 = lean_nat_dec_le(x_19, x_19); -if (x_24 == 0) +lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; uint8_t x_52; lean_object* x_53; uint8_t x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_41 = lean_ctor_get(x_9, 0); +x_42 = lean_ctor_get(x_9, 1); +x_43 = lean_ctor_get(x_9, 2); +x_44 = lean_ctor_get(x_9, 3); +x_45 = lean_ctor_get(x_9, 4); +x_46 = lean_ctor_get(x_9, 5); +x_47 = lean_ctor_get(x_9, 6); +x_48 = lean_ctor_get(x_9, 7); +x_49 = lean_ctor_get(x_9, 8); +x_50 = lean_ctor_get(x_9, 9); +x_51 = lean_ctor_get(x_9, 10); +x_52 = lean_ctor_get_uint8(x_9, sizeof(void*)*12); +x_53 = lean_ctor_get(x_9, 11); +x_54 = lean_ctor_get_uint8(x_9, sizeof(void*)*12 + 1); +lean_inc(x_53); +lean_inc(x_51); +lean_inc(x_50); +lean_inc(x_49); +lean_inc(x_48); +lean_inc(x_47); +lean_inc(x_46); +lean_inc(x_45); +lean_inc(x_44); +lean_inc(x_43); +lean_inc(x_42); +lean_inc(x_41); +lean_dec(x_9); +x_55 = l_Lean_replaceRef(x_1, x_46); +lean_dec(x_46); +x_56 = lean_alloc_ctor(0, 12, 2); +lean_ctor_set(x_56, 0, x_41); +lean_ctor_set(x_56, 1, x_42); +lean_ctor_set(x_56, 2, x_43); +lean_ctor_set(x_56, 3, x_44); +lean_ctor_set(x_56, 4, x_45); +lean_ctor_set(x_56, 5, x_55); +lean_ctor_set(x_56, 6, x_47); +lean_ctor_set(x_56, 7, x_48); +lean_ctor_set(x_56, 8, x_49); +lean_ctor_set(x_56, 9, x_50); +lean_ctor_set(x_56, 10, x_51); +lean_ctor_set(x_56, 11, x_53); +lean_ctor_set_uint8(x_56, sizeof(void*)*12, x_52); +lean_ctor_set_uint8(x_56, sizeof(void*)*12 + 1, x_54); +lean_inc(x_10); +lean_inc(x_56); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_3); +x_57 = l_Lean_Elab_Command_mkStructureDecl(x_2, x_3, x_5, x_6, x_7, x_8, x_56, x_10, x_11); +if (lean_obj_tag(x_57) == 0) +{ +uint8_t x_58; +x_58 = lean_ctor_get_uint8(x_3, sizeof(void*)*12); +lean_dec(x_3); +if (x_58 == 0) { -lean_object* x_25; lean_object* x_26; -lean_dec(x_19); -x_25 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabStructure___lambda__6___boxed), 10, 2); -lean_closure_set(x_25, 0, x_2); -lean_closure_set(x_25, 1, x_17); -x_26 = l_Lean_Elab_Command_runTermElabM___rarg(x_25, x_10, x_11, x_18); -lean_dec(x_11); -lean_dec(x_10); -return x_26; -} -else +lean_object* x_59; lean_object* x_60; +x_59 = lean_ctor_get(x_57, 1); +lean_inc(x_59); +lean_dec(x_57); +lean_inc(x_10); +lean_inc(x_56); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_4); +x_60 = l_Lean_Meta_IndPredBelow_mkBelow(x_4, x_7, x_8, x_56, x_10, x_59); +if (lean_obj_tag(x_60) == 0) { -size_t x_27; size_t x_28; lean_object* x_29; lean_object* x_30; -x_27 = 0; -x_28 = lean_usize_of_nat(x_19); -lean_dec(x_19); -x_29 = lean_box(0); -lean_inc(x_11); +lean_object* x_61; lean_object* x_62; +x_61 = lean_ctor_get(x_60, 1); +lean_inc(x_61); +lean_dec(x_60); lean_inc(x_10); -lean_inc(x_17); -x_30 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabStructure___spec__3(x_17, x_8, x_27, x_28, x_29, x_10, x_11, x_18); -if (lean_obj_tag(x_30) == 0) +lean_inc(x_56); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_4); +x_62 = l_Lean_Meta_mkSizeOfInstances(x_4, x_7, x_8, x_56, x_10, x_61); +if (lean_obj_tag(x_62) == 0) { -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 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabStructure___lambda__6___boxed), 10, 2); -lean_closure_set(x_32, 0, x_2); -lean_closure_set(x_32, 1, x_17); -x_33 = l_Lean_Elab_Command_runTermElabM___rarg(x_32, x_10, x_11, x_31); -lean_dec(x_11); -lean_dec(x_10); -return x_33; +lean_object* x_63; lean_object* x_64; +x_63 = lean_ctor_get(x_62, 1); +lean_inc(x_63); +lean_dec(x_62); +x_64 = l_Lean_Meta_mkInjectiveTheorems(x_4, x_7, x_8, x_56, x_10, x_63); +return x_64; } else { -uint8_t x_34; -lean_dec(x_17); -lean_dec(x_11); +lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; +lean_dec(x_56); lean_dec(x_10); -lean_dec(x_2); -x_34 = !lean_is_exclusive(x_30); -if (x_34 == 0) -{ -return x_30; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_4); +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; +} else { + lean_dec_ref(x_62); + x_67 = lean_box(0); +} +if (lean_is_scalar(x_67)) { + x_68 = lean_alloc_ctor(1, 2, 0); +} else { + x_68 = x_67; +} +lean_ctor_set(x_68, 0, x_65); +lean_ctor_set(x_68, 1, x_66); +return x_68; +} } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_35 = lean_ctor_get(x_30, 0); -x_36 = lean_ctor_get(x_30, 1); -lean_inc(x_36); -lean_inc(x_35); -lean_dec(x_30); -x_37 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -return x_37; -} +lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; +lean_dec(x_56); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_4); +x_69 = lean_ctor_get(x_60, 0); +lean_inc(x_69); +x_70 = lean_ctor_get(x_60, 1); +lean_inc(x_70); +if (lean_is_exclusive(x_60)) { + lean_ctor_release(x_60, 0); + lean_ctor_release(x_60, 1); + x_71 = x_60; +} else { + lean_dec_ref(x_60); + 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_38; -lean_dec(x_11); +lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; +lean_dec(x_56); lean_dec(x_10); -lean_dec(x_2); -x_38 = !lean_is_exclusive(x_16); -if (x_38 == 0) -{ -return x_16; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_4); +x_73 = lean_ctor_get(x_57, 1); +lean_inc(x_73); +if (lean_is_exclusive(x_57)) { + lean_ctor_release(x_57, 0); + lean_ctor_release(x_57, 1); + x_74 = x_57; +} else { + lean_dec_ref(x_57); + x_74 = lean_box(0); +} +x_75 = lean_box(0); +if (lean_is_scalar(x_74)) { + x_76 = lean_alloc_ctor(0, 2, 0); +} else { + x_76 = x_74; +} +lean_ctor_set(x_76, 0, x_75); +lean_ctor_set(x_76, 1, x_73); +return x_76; +} } else { -lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_39 = lean_ctor_get(x_16, 0); -x_40 = lean_ctor_get(x_16, 1); -lean_inc(x_40); -lean_inc(x_39); -lean_dec(x_16); -x_41 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_41, 0, x_39); -lean_ctor_set(x_41, 1, x_40); -return x_41; +lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; +lean_dec(x_56); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_4); +lean_dec(x_3); +x_77 = lean_ctor_get(x_57, 0); +lean_inc(x_77); +x_78 = lean_ctor_get(x_57, 1); +lean_inc(x_78); +if (lean_is_exclusive(x_57)) { + lean_ctor_release(x_57, 0); + lean_ctor_release(x_57, 1); + x_79 = x_57; +} else { + lean_dec_ref(x_57); + 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; } } -static lean_object* _init_l_Lean_Elab_Command_elabStructure___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("sort", 4, 4); -return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_elabStructure___closed__2() { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructureView(lean_object* x_1, lean_object* x_2, lean_object* x_3, 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; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__1; -x_2 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__2; -x_3 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__3; -x_4 = l_Lean_Elab_Command_elabStructure___closed__1; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_10 = lean_ctor_get(x_2, 4); +lean_inc(x_10); +x_11 = lean_ctor_get(x_2, 0); +lean_inc(x_11); +lean_inc(x_10); +x_12 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabStructureView___lambda__1___boxed), 11, 4); +lean_closure_set(x_12, 0, x_11); +lean_closure_set(x_12, 1, x_1); +lean_closure_set(x_12, 2, x_2); +lean_closure_set(x_12, 3, x_10); +x_13 = l_Lean_Elab_Term_withDeclName___rarg(x_10, x_12, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_13; } } -static lean_object* _init_l_Lean_Elab_Command_elabStructure___closed__3() { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructureView___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Sort", 4, 4); -return x_1; +lean_object* x_12; +x_12 = l_Lean_Elab_Command_elabStructureView___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_1); +return x_12; } } -static lean_object* _init_l_Lean_Elab_Command_elabStructure___closed__4() { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabStructureViewPostprocessing___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) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Level", 5, 5); -return x_1; +uint8_t x_9; +x_9 = lean_usize_dec_eq(x_3, x_4); +if (x_9 == 0) +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_dec(x_5); +x_10 = lean_array_uget(x_2, x_3); +x_11 = lean_ctor_get(x_1, 4); +x_12 = lean_box(0); +lean_inc(x_11); +x_13 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_13, 0, x_11); +lean_ctor_set(x_13, 1, x_12); +x_14 = lean_array_mk(x_13); +lean_inc(x_7); +lean_inc(x_6); +x_15 = l_Lean_Elab_DerivingClassView_applyHandlers(x_10, x_14, x_6, x_7, x_8); +if (lean_obj_tag(x_15) == 0) +{ +lean_object* x_16; lean_object* x_17; size_t x_18; size_t 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 = 1; +x_19 = lean_usize_add(x_3, x_18); +x_3 = x_19; +x_5 = x_16; +x_8 = x_17; +goto _start; } +else +{ +uint8_t x_21; +lean_dec(x_7); +lean_dec(x_6); +x_21 = !lean_is_exclusive(x_15); +if (x_21 == 0) +{ +return x_15; } -static lean_object* _init_l_Lean_Elab_Command_elabStructure___closed__5() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("hole", 4, 4); -return x_1; +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_15, 0); +x_23 = lean_ctor_get(x_15, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_15); +x_24 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); +return x_24; } } -static lean_object* _init_l_Lean_Elab_Command_elabStructure___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_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__1; -x_2 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__2; -x_3 = l_Lean_Elab_Command_elabStructure___closed__4; -x_4 = l_Lean_Elab_Command_elabStructure___closed__5; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; +lean_object* x_25; +lean_dec(x_7); +lean_dec(x_6); +x_25 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_25, 0, x_5); +lean_ctor_set(x_25, 1, x_8); +return x_25; } } -static lean_object* _init_l_Lean_Elab_Command_elabStructure___closed__7() { +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructureViewPostprocessing___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("_", 1, 1); -return x_1; +uint8_t x_11; +x_11 = !lean_is_exclusive(x_8); +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_8, 5); +x_13 = l_Lean_replaceRef(x_1, x_12); +lean_dec(x_12); +lean_ctor_set(x_8, 5, x_13); +x_14 = 1; +x_15 = l_Lean_Elab_Term_applyAttributesAt(x_2, x_3, x_14, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_15; } +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; lean_object* x_28; uint8_t x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; lean_object* x_33; +x_16 = lean_ctor_get(x_8, 0); +x_17 = lean_ctor_get(x_8, 1); +x_18 = lean_ctor_get(x_8, 2); +x_19 = lean_ctor_get(x_8, 3); +x_20 = lean_ctor_get(x_8, 4); +x_21 = lean_ctor_get(x_8, 5); +x_22 = lean_ctor_get(x_8, 6); +x_23 = lean_ctor_get(x_8, 7); +x_24 = lean_ctor_get(x_8, 8); +x_25 = lean_ctor_get(x_8, 9); +x_26 = lean_ctor_get(x_8, 10); +x_27 = lean_ctor_get_uint8(x_8, sizeof(void*)*12); +x_28 = lean_ctor_get(x_8, 11); +x_29 = lean_ctor_get_uint8(x_8, sizeof(void*)*12 + 1); +lean_inc(x_28); +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_8); +x_30 = l_Lean_replaceRef(x_1, x_21); +lean_dec(x_21); +x_31 = lean_alloc_ctor(0, 12, 2); +lean_ctor_set(x_31, 0, x_16); +lean_ctor_set(x_31, 1, x_17); +lean_ctor_set(x_31, 2, x_18); +lean_ctor_set(x_31, 3, x_19); +lean_ctor_set(x_31, 4, x_20); +lean_ctor_set(x_31, 5, x_30); +lean_ctor_set(x_31, 6, x_22); +lean_ctor_set(x_31, 7, x_23); +lean_ctor_set(x_31, 8, x_24); +lean_ctor_set(x_31, 9, x_25); +lean_ctor_set(x_31, 10, x_26); +lean_ctor_set(x_31, 11, x_28); +lean_ctor_set_uint8(x_31, sizeof(void*)*12, x_27); +lean_ctor_set_uint8(x_31, sizeof(void*)*12 + 1, x_29); +x_32 = 1; +x_33 = l_Lean_Elab_Term_applyAttributesAt(x_2, x_3, x_32, x_4, x_5, x_6, x_7, x_31, x_9, x_10); +return x_33; } -static lean_object* _init_l_Lean_Elab_Command_elabStructure___closed__8() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__14; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_elabStructure___closed__9() { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructureViewPostprocessing___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -uint8_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = 0; -x_2 = l_Lean_Elab_Command_elabStructure___closed__8; -x_3 = lean_box(0); -x_4 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_4, 0, x_2); -lean_ctor_set(x_4, 1, x_3); -lean_ctor_set_uint8(x_4, sizeof(void*)*2, x_1); -return x_4; +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_10 = lean_ctor_get(x_1, 4); +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); +lean_dec(x_1); +x_13 = lean_ctor_get(x_12, 2); +lean_inc(x_13); +lean_dec(x_12); +lean_inc(x_10); +x_14 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabStructureViewPostprocessing___lambda__1___boxed), 10, 3); +lean_closure_set(x_14, 0, x_11); +lean_closure_set(x_14, 1, x_10); +lean_closure_set(x_14, 2, x_13); +x_15 = l_Lean_Elab_Term_withDeclName___rarg(x_10, x_14, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_15; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructureViewPostprocessing(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_6; -lean_inc(x_3); -x_6 = l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1(x_1, x_3, x_4, x_5); -if (lean_obj_tag(x_6) == 0) +lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; +x_5 = lean_ctor_get(x_1, 11); +lean_inc(x_5); +x_6 = lean_array_get_size(x_5); +x_7 = lean_unsigned_to_nat(0u); +x_8 = lean_nat_dec_lt(x_7, x_6); +if (x_8 == 0) { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; -x_7 = lean_ctor_get(x_6, 1); -lean_inc(x_7); +lean_object* x_9; lean_object* x_10; lean_dec(x_6); -x_8 = lean_unsigned_to_nat(0u); -x_9 = l_Lean_Syntax_getArg(x_2, x_8); -x_10 = l_Lean_Syntax_getKind(x_9); -x_11 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__3; -x_12 = lean_name_eq(x_10, x_11); -lean_dec(x_10); -x_13 = lean_unsigned_to_nat(1u); -x_14 = l_Lean_Syntax_getArg(x_2, x_13); -x_15 = lean_unsigned_to_nat(2u); -x_16 = l_Lean_Syntax_getArg(x_2, x_15); -x_17 = l_Lean_Syntax_getArgs(x_16); -lean_dec(x_16); -x_18 = lean_unsigned_to_nat(3u); -x_19 = l_Lean_Syntax_getArg(x_2, x_18); -x_20 = l_Lean_Syntax_isNone(x_19); -x_21 = lean_unsigned_to_nat(4u); -x_22 = l_Lean_Syntax_getArg(x_2, x_21); -x_23 = lean_unsigned_to_nat(6u); -x_24 = l_Lean_Syntax_getArg(x_2, x_23); -x_25 = lean_alloc_closure((void*)(l_Lean_Elab_getOptDerivingClasses), 4, 1); -lean_closure_set(x_25, 0, x_24); -x_26 = l_Lean_Elab_Command_liftCoreM___rarg(x_25, x_3, x_4, x_7); -if (x_12 == 0) -{ -uint8_t x_105; -x_105 = 0; -x_27 = x_105; -goto block_104; +lean_dec(x_5); +x_9 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabStructureViewPostprocessing___lambda__2___boxed), 9, 1); +lean_closure_set(x_9, 0, x_1); +x_10 = l_Lean_Elab_Command_runTermElabM___rarg(x_9, x_2, x_3, x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_10; } else { -uint8_t x_106; -x_106 = 1; -x_27 = x_106; -goto block_104; -} -block_104: -{ -lean_object* x_28; -if (x_27 == 0) +uint8_t x_11; +x_11 = lean_nat_dec_le(x_6, x_6); +if (x_11 == 0) { -x_28 = x_1; -goto block_101; +lean_object* x_12; lean_object* x_13; +lean_dec(x_6); +lean_dec(x_5); +x_12 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabStructureViewPostprocessing___lambda__2___boxed), 9, 1); +lean_closure_set(x_12, 0, x_1); +x_13 = l_Lean_Elab_Command_runTermElabM___rarg(x_12, x_2, x_3, x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_13; } else { -lean_object* x_102; lean_object* x_103; -x_102 = l_Lean_Elab_Command_elabStructure___closed__9; -x_103 = l_Lean_Elab_Modifiers_addAttr(x_1, x_102); -x_28 = x_103; -goto block_101; -} -block_101: -{ -lean_object* x_29; lean_object* x_30; lean_object* x_31; -if (x_20 == 0) -{ -if (lean_obj_tag(x_26) == 0) +size_t x_14; size_t x_15; lean_object* x_16; lean_object* x_17; +x_14 = 0; +x_15 = lean_usize_of_nat(x_6); +lean_dec(x_6); +x_16 = lean_box(0); +lean_inc(x_3); +lean_inc(x_2); +x_17 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabStructureViewPostprocessing___spec__1(x_1, x_5, x_14, x_15, x_16, x_2, x_3, x_4); +lean_dec(x_5); +if (lean_obj_tag(x_17) == 0) { -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_26, 0); -lean_inc(x_85); -x_86 = lean_ctor_get(x_26, 1); -lean_inc(x_86); -lean_dec(x_26); -x_87 = l_Lean_Syntax_getArg(x_19, x_8); -lean_dec(x_19); -x_88 = l_Lean_Syntax_getArg(x_87, x_13); -lean_dec(x_87); -x_89 = l_Lean_Syntax_getSepArgs(x_88); -lean_dec(x_88); -x_29 = x_89; -x_30 = x_85; -x_31 = x_86; -goto block_84; +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_17, 1); +lean_inc(x_18); +lean_dec(x_17); +x_19 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabStructureViewPostprocessing___lambda__2___boxed), 9, 1); +lean_closure_set(x_19, 0, x_1); +x_20 = l_Lean_Elab_Command_runTermElabM___rarg(x_19, x_2, x_3, x_18); +lean_dec(x_3); +lean_dec(x_2); +return x_20; } else { -uint8_t x_90; -lean_dec(x_28); -lean_dec(x_22); -lean_dec(x_19); -lean_dec(x_17); -lean_dec(x_14); -lean_dec(x_4); +uint8_t x_21; lean_dec(x_3); lean_dec(x_2); -x_90 = !lean_is_exclusive(x_26); -if (x_90 == 0) +lean_dec(x_1); +x_21 = !lean_is_exclusive(x_17); +if (x_21 == 0) { -return x_26; +return x_17; } else { -lean_object* x_91; lean_object* x_92; lean_object* x_93; -x_91 = lean_ctor_get(x_26, 0); -x_92 = lean_ctor_get(x_26, 1); -lean_inc(x_92); -lean_inc(x_91); -lean_dec(x_26); -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_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_17, 0); +x_23 = lean_ctor_get(x_17, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_17); +x_24 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); +return x_24; } } } -else -{ -lean_dec(x_19); -if (lean_obj_tag(x_26) == 0) -{ -lean_object* x_94; lean_object* x_95; lean_object* x_96; -x_94 = lean_ctor_get(x_26, 0); -lean_inc(x_94); -x_95 = lean_ctor_get(x_26, 1); -lean_inc(x_95); -lean_dec(x_26); -x_96 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; -x_29 = x_96; -x_30 = x_94; -x_31 = x_95; -goto block_84; } -else +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabStructureViewPostprocessing___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: { -uint8_t x_97; -lean_dec(x_28); -lean_dec(x_22); -lean_dec(x_17); -lean_dec(x_14); -lean_dec(x_4); +size_t x_9; size_t x_10; lean_object* x_11; +x_9 = lean_unbox_usize(x_3); lean_dec(x_3); +x_10 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_11 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabStructureViewPostprocessing___spec__1(x_1, x_2, x_9, x_10, x_5, x_6, x_7, x_8); lean_dec(x_2); -x_97 = !lean_is_exclusive(x_26); -if (x_97 == 0) -{ -return x_26; +lean_dec(x_1); +return x_11; } -else -{ -lean_object* x_98; lean_object* x_99; lean_object* x_100; -x_98 = lean_ctor_get(x_26, 0); -x_99 = lean_ctor_get(x_26, 1); -lean_inc(x_99); -lean_inc(x_98); -lean_dec(x_26); -x_100 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_100, 0, x_98); -lean_ctor_set(x_100, 1, x_99); -return x_100; } +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructureViewPostprocessing___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, 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_Command_elabStructureViewPostprocessing___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_1); +return x_11; } } -block_84: -{ -uint8_t x_32; -x_32 = l_Lean_Syntax_isNone(x_22); -if (x_32 == 0) +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructureViewPostprocessing___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_33; lean_object* x_34; lean_object* x_35; -x_33 = l_Lean_Syntax_getArg(x_22, x_8); -lean_dec(x_22); -x_34 = l_Lean_Syntax_getArg(x_33, x_13); -lean_dec(x_33); -x_35 = l_Lean_Elab_Command_elabStructure___lambda__7(x_14, x_28, x_2, x_12, x_29, x_27, x_17, x_30, x_34, x_3, x_4, x_31); -lean_dec(x_30); -return x_35; +lean_object* x_10; +x_10 = l_Lean_Elab_Command_elabStructureViewPostprocessing___lambda__2(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; } -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; uint8_t x_42; -lean_dec(x_22); -x_36 = l_Lean_Elab_Command_getRef(x_3, x_4, x_31); -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 = 0; -x_40 = l_Lean_SourceInfo_fromRef(x_37, x_39); -lean_dec(x_37); -x_41 = l_Lean_Elab_Command_getCurrMacroScope(x_3, x_4, x_38); -x_42 = !lean_is_exclusive(x_41); -if (x_42 == 0) +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___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_43; lean_object* x_44; lean_object* x_45; uint8_t x_46; -x_43 = lean_ctor_get(x_41, 1); -x_44 = lean_ctor_get(x_41, 0); -lean_dec(x_44); -x_45 = l_Lean_Elab_Command_getMainModule___rarg(x_4, x_43); -x_46 = !lean_is_exclusive(x_45); -if (x_46 == 0) +lean_object* x_11; +lean_inc(x_2); +x_11 = l_Lean_Elab_Command_elabStructureView(x_1, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_11) == 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; -x_47 = lean_ctor_get(x_45, 1); -x_48 = lean_ctor_get(x_45, 0); -lean_dec(x_48); -x_49 = l_Lean_Elab_Command_elabStructure___closed__3; -lean_inc(x_40); -lean_ctor_set_tag(x_45, 2); -lean_ctor_set(x_45, 1, x_49); -lean_ctor_set(x_45, 0, x_40); -x_50 = l_Lean_Elab_Command_elabStructure___closed__7; -lean_inc(x_40); -lean_ctor_set_tag(x_41, 2); -lean_ctor_set(x_41, 1, x_50); -lean_ctor_set(x_41, 0, x_40); -x_51 = l_Lean_Elab_Command_elabStructure___closed__6; -lean_inc(x_40); -x_52 = l_Lean_Syntax_node1(x_40, x_51, x_41); -x_53 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__6; -lean_inc(x_40); -x_54 = l_Lean_Syntax_node1(x_40, x_53, x_52); -x_55 = l_Lean_Elab_Command_elabStructure___closed__2; -x_56 = l_Lean_Syntax_node2(x_40, x_55, x_45, x_54); -x_57 = l_Lean_Elab_Command_elabStructure___lambda__7(x_14, x_28, x_2, x_12, x_29, x_27, x_17, x_30, x_56, x_3, x_4, x_47); -lean_dec(x_30); -return x_57; -} -else +uint8_t x_12; +x_12 = !lean_is_exclusive(x_11); +if (x_12 == 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; -x_58 = lean_ctor_get(x_45, 1); -lean_inc(x_58); -lean_dec(x_45); -x_59 = l_Lean_Elab_Command_elabStructure___closed__3; -lean_inc(x_40); -x_60 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_60, 0, x_40); -lean_ctor_set(x_60, 1, x_59); -x_61 = l_Lean_Elab_Command_elabStructure___closed__7; -lean_inc(x_40); -lean_ctor_set_tag(x_41, 2); -lean_ctor_set(x_41, 1, x_61); -lean_ctor_set(x_41, 0, x_40); -x_62 = l_Lean_Elab_Command_elabStructure___closed__6; -lean_inc(x_40); -x_63 = l_Lean_Syntax_node1(x_40, x_62, x_41); -x_64 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__6; -lean_inc(x_40); -x_65 = l_Lean_Syntax_node1(x_40, x_64, x_63); -x_66 = l_Lean_Elab_Command_elabStructure___closed__2; -x_67 = l_Lean_Syntax_node2(x_40, x_66, x_60, x_65); -x_68 = l_Lean_Elab_Command_elabStructure___lambda__7(x_14, x_28, x_2, x_12, x_29, x_27, x_17, x_30, x_67, x_3, x_4, x_58); -lean_dec(x_30); -return x_68; -} +lean_object* x_13; +x_13 = lean_ctor_get(x_11, 0); +lean_dec(x_13); +lean_ctor_set(x_11, 0, x_2); +return x_11; } else { -lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; -x_69 = lean_ctor_get(x_41, 1); -lean_inc(x_69); -lean_dec(x_41); -x_70 = l_Lean_Elab_Command_getMainModule___rarg(x_4, 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_70); - x_72 = lean_box(0); -} -x_73 = l_Lean_Elab_Command_elabStructure___closed__3; -lean_inc(x_40); -if (lean_is_scalar(x_72)) { - x_74 = lean_alloc_ctor(2, 2, 0); -} else { - x_74 = x_72; - lean_ctor_set_tag(x_74, 2); -} -lean_ctor_set(x_74, 0, x_40); -lean_ctor_set(x_74, 1, x_73); -x_75 = l_Lean_Elab_Command_elabStructure___closed__7; -lean_inc(x_40); -x_76 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_76, 0, x_40); -lean_ctor_set(x_76, 1, x_75); -x_77 = l_Lean_Elab_Command_elabStructure___closed__6; -lean_inc(x_40); -x_78 = l_Lean_Syntax_node1(x_40, x_77, x_76); -x_79 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__6; -lean_inc(x_40); -x_80 = l_Lean_Syntax_node1(x_40, x_79, x_78); -x_81 = l_Lean_Elab_Command_elabStructure___closed__2; -x_82 = l_Lean_Syntax_node2(x_40, x_81, x_74, x_80); -x_83 = l_Lean_Elab_Command_elabStructure___lambda__7(x_14, x_28, x_2, x_12, x_29, x_27, x_17, x_30, x_82, x_3, x_4, x_71); -lean_dec(x_30); -return x_83; -} -} -} -} +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_11, 1); +lean_inc(x_14); +lean_dec(x_11); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_2); +lean_ctor_set(x_15, 1, x_14); +return x_15; } } else { -uint8_t x_107; -lean_dec(x_4); -lean_dec(x_3); +uint8_t x_16; lean_dec(x_2); -lean_dec(x_1); -x_107 = !lean_is_exclusive(x_6); -if (x_107 == 0) +x_16 = !lean_is_exclusive(x_11); +if (x_16 == 0) { -return x_6; +return x_11; } else { -lean_object* x_108; lean_object* x_109; lean_object* x_110; -x_108 = lean_ctor_get(x_6, 0); -x_109 = lean_ctor_get(x_6, 1); -lean_inc(x_109); -lean_inc(x_108); -lean_dec(x_6); -x_110 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_110, 0, x_108); -lean_ctor_set(x_110, 1, x_109); -return x_110; +lean_object* x_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_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___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) { +static lean_object* _init_l_Lean_Elab_Command_elabStructure___lambda__2___closed__1() { _start: { -lean_object* x_6; -x_6 = l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1___lambda__1(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_object* x_1; +x_1 = lean_mk_string_unchecked("view.levelNames: ", 17, 17); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +static lean_object* _init_l_Lean_Elab_Command_elabStructure___lambda__2___closed__2() { _start: { -lean_object* x_5; -x_5 = l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1(x_1, x_2, x_3, x_4); -lean_dec(x_3); -lean_dec(x_1); -return x_5; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_elabStructure___lambda__2___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___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_10; -x_10 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_8); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -return x_10; +lean_object* x_11; +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_11 = l_Lean_Elab_Command_structureSyntaxToView(x_1, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_11) == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +x_14 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__1; +x_15 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_14, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +x_17 = lean_unbox(x_16); +lean_dec(x_16); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_15, 1); +lean_inc(x_18); +lean_dec(x_15); +x_19 = lean_box(0); +x_20 = l_Lean_Elab_Command_elabStructure___lambda__1(x_3, x_12, x_19, x_4, x_5, x_6, x_7, x_8, x_9, x_18); +return x_20; } +else +{ +uint8_t x_21; +x_21 = !lean_is_exclusive(x_15); +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; +x_22 = lean_ctor_get(x_15, 1); +x_23 = lean_ctor_get(x_15, 0); +lean_dec(x_23); +x_24 = lean_ctor_get(x_12, 5); +lean_inc(x_24); +x_25 = lean_box(0); +x_26 = l_List_mapTR_loop___at_Lean_compileDecl___spec__1(x_24, x_25); +x_27 = l_Lean_MessageData_ofList(x_26); +x_28 = l_Lean_Elab_Command_elabStructure___lambda__2___closed__2; +lean_ctor_set_tag(x_15, 7); +lean_ctor_set(x_15, 1, x_27); +lean_ctor_set(x_15, 0, x_28); +x_29 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3; +x_30 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_30, 0, x_15); +lean_ctor_set(x_30, 1, x_29); +x_31 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_14, x_30, x_4, x_5, x_6, x_7, x_8, x_9, x_22); +x_32 = lean_ctor_get(x_31, 0); +lean_inc(x_32); +x_33 = lean_ctor_get(x_31, 1); +lean_inc(x_33); +lean_dec(x_31); +x_34 = l_Lean_Elab_Command_elabStructure___lambda__1(x_3, x_12, x_32, x_4, x_5, x_6, x_7, x_8, x_9, x_33); +lean_dec(x_32); +return x_34; } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabStructure___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: +else { -size_t x_9; size_t x_10; lean_object* x_11; -x_9 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_10 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_11 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabStructure___spec__3(x_1, x_2, x_9, x_10, x_5, x_6, x_7, x_8); -lean_dec(x_2); -return x_11; +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_35 = lean_ctor_get(x_15, 1); +lean_inc(x_35); +lean_dec(x_15); +x_36 = lean_ctor_get(x_12, 5); +lean_inc(x_36); +x_37 = lean_box(0); +x_38 = l_List_mapTR_loop___at_Lean_compileDecl___spec__1(x_36, x_37); +x_39 = l_Lean_MessageData_ofList(x_38); +x_40 = l_Lean_Elab_Command_elabStructure___lambda__2___closed__2; +x_41 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_41, 0, x_40); +lean_ctor_set(x_41, 1, x_39); +x_42 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3; +x_43 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_43, 0, x_41); +lean_ctor_set(x_43, 1, x_42); +x_44 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_14, x_43, x_4, x_5, x_6, x_7, x_8, x_9, x_35); +x_45 = lean_ctor_get(x_44, 0); +lean_inc(x_45); +x_46 = lean_ctor_get(x_44, 1); +lean_inc(x_46); +lean_dec(x_44); +x_47 = l_Lean_Elab_Command_elabStructure___lambda__1(x_3, x_12, x_45, x_4, x_5, x_6, x_7, x_8, x_9, x_46); +lean_dec(x_45); +return x_47; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +} +else { -lean_object* x_10; -x_10 = l_Lean_Elab_Command_elabStructure___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +uint8_t x_48; +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); -return x_10; -} +x_48 = !lean_is_exclusive(x_11); +if (x_48 == 0) +{ +return x_11; } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___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]; -_start: +else { -uint8_t x_20; uint8_t x_21; lean_object* x_22; -x_20 = lean_unbox(x_4); -lean_dec(x_4); -x_21 = lean_unbox(x_11); +lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_49 = lean_ctor_get(x_11, 0); +x_50 = lean_ctor_get(x_11, 1); +lean_inc(x_50); +lean_inc(x_49); lean_dec(x_11); -x_22 = l_Lean_Elab_Command_elabStructure___lambda__2(x_1, x_2, x_3, x_20, x_5, x_6, x_7, x_8, x_9, x_10, x_21, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19); -lean_dec(x_12); -return x_22; +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_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___lambda__3___boxed(lean_object** _args) { -lean_object* x_1 = _args[0]; -lean_object* x_2 = _args[1]; -lean_object* x_3 = _args[2]; -lean_object* x_4 = _args[3]; -lean_object* x_5 = _args[4]; -lean_object* x_6 = _args[5]; -lean_object* x_7 = _args[6]; -lean_object* x_8 = _args[7]; -lean_object* x_9 = _args[8]; -lean_object* x_10 = _args[9]; -lean_object* x_11 = _args[10]; -lean_object* x_12 = _args[11]; -lean_object* x_13 = _args[12]; -lean_object* x_14 = _args[13]; -lean_object* x_15 = _args[14]; -lean_object* x_16 = _args[15]; -lean_object* x_17 = _args[16]; -lean_object* x_18 = _args[17]; -_start: -{ -uint8_t x_19; uint8_t x_20; lean_object* x_21; -x_19 = lean_unbox(x_5); -lean_dec(x_5); -x_20 = lean_unbox(x_9); -lean_dec(x_9); -x_21 = l_Lean_Elab_Command_elabStructure___lambda__3(x_1, x_2, x_3, x_4, x_19, x_6, x_7, x_8, x_20, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18); -return x_21; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___lambda__4___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_EXPORT lean_object* l_Lean_Elab_Command_elabStructure(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -uint8_t x_19; uint8_t x_20; lean_object* x_21; -x_19 = lean_unbox(x_5); -lean_dec(x_5); -x_20 = lean_unbox(x_9); -lean_dec(x_9); -x_21 = l_Lean_Elab_Command_elabStructure___lambda__4(x_1, x_2, x_3, x_4, x_19, x_6, x_7, x_8, x_20, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18); -return x_21; -} +lean_object* x_6; lean_object* x_7; +x_6 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabStructure___lambda__2), 10, 2); +lean_closure_set(x_6, 0, x_1); +lean_closure_set(x_6, 1, x_2); +x_7 = l_Lean_Elab_Command_runTermElabM___rarg(x_6, x_3, x_4, x_5); +if (lean_obj_tag(x_7) == 0) +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; +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_Elab_Command_elabStructureViewPostprocessing(x_8, x_3, x_4, x_9); +return x_10; } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: +else { -uint8_t x_17; uint8_t x_18; lean_object* x_19; -x_17 = lean_unbox(x_4); +uint8_t x_11; lean_dec(x_4); -x_18 = lean_unbox(x_7); +lean_dec(x_3); +x_11 = !lean_is_exclusive(x_7); +if (x_11 == 0) +{ +return x_7; +} +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_7, 0); +x_13 = lean_ctor_get(x_7, 1); +lean_inc(x_13); +lean_inc(x_12); lean_dec(x_7); -x_19 = l_Lean_Elab_Command_elabStructure___lambda__5(x_1, x_2, x_3, x_17, x_5, x_6, x_18, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_1); -return x_19; +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_Command_elabStructure___lambda__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, 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_Command_elabStructure___lambda__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Lean_Elab_Command_elabStructure___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_3); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -uint8_t x_13; uint8_t x_14; lean_object* x_15; -x_13 = lean_unbox(x_4); -lean_dec(x_4); -x_14 = lean_unbox(x_6); -lean_dec(x_6); -x_15 = l_Lean_Elab_Command_elabStructure___lambda__7(x_1, x_2, x_3, x_13, x_5, x_14, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_8); -return x_15; -} -} -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__1() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____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_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__1; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__2() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__1; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__1; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__7; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__3() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__2; -x_2 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__1; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__2; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__8; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__4() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__4() { _start: { lean_object* x_1; @@ -35364,17 +34490,17 @@ x_1 = lean_mk_string_unchecked("initFn", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__5() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__3; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__4; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__3; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__4; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__6() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__6() { _start: { lean_object* x_1; @@ -35382,37 +34508,37 @@ x_1 = lean_mk_string_unchecked("_@", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__7() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__5; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__6; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__5; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__8() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__7; -x_2 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__1; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__7; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__9() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__8; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__8; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__7; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__10() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__10() { _start: { lean_object* x_1; @@ -35420,17 +34546,17 @@ x_1 = lean_mk_string_unchecked("Structure", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__11() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__9; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__10; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__9; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__10; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__12() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__12() { _start: { lean_object* x_1; @@ -35438,33 +34564,33 @@ x_1 = lean_mk_string_unchecked("_hyg", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__13() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__11; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__12; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__11; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__12; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__14() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__13; -x_2 = lean_unsigned_to_nat(14022u); +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__13; +x_2 = lean_unsigned_to_nat(15311u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311_(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; -x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__4___closed__1; +x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__1; x_3 = 0; -x_4 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__14; +x_4 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__14; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); return x_5; } @@ -35526,235 +34652,191 @@ lean_dec_ref(res); res = initialize_Lean_Elab_Binders(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__1 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__1(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__1); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__2 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__2(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__2); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__3 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__3(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__3); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__4 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__4(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__4); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__5 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__5(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__5); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__6 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__6(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__6); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__7 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__7(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__7); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__8 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__8(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__8); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__9 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__9(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5____closed__9); +if (builtin) {res = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_5_(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +l_Lean_Elab_Command_structureDiamondWarning = lean_io_result_get_value(res); +lean_mark_persistent(l_Lean_Elab_Command_structureDiamondWarning); +lean_dec_ref(res); +}l_Lean_Elab_Command_instInhabitedStructCtorView___closed__1 = _init_l_Lean_Elab_Command_instInhabitedStructCtorView___closed__1(); +lean_mark_persistent(l_Lean_Elab_Command_instInhabitedStructCtorView___closed__1); +l_Lean_Elab_Command_instInhabitedStructCtorView___closed__2 = _init_l_Lean_Elab_Command_instInhabitedStructCtorView___closed__2(); +lean_mark_persistent(l_Lean_Elab_Command_instInhabitedStructCtorView___closed__2); +l_Lean_Elab_Command_instInhabitedStructCtorView___closed__3 = _init_l_Lean_Elab_Command_instInhabitedStructCtorView___closed__3(); +lean_mark_persistent(l_Lean_Elab_Command_instInhabitedStructCtorView___closed__3); +l_Lean_Elab_Command_instInhabitedStructCtorView = _init_l_Lean_Elab_Command_instInhabitedStructCtorView(); +lean_mark_persistent(l_Lean_Elab_Command_instInhabitedStructCtorView); +l_Lean_Elab_Command_instInhabitedStructView___closed__1 = _init_l_Lean_Elab_Command_instInhabitedStructView___closed__1(); +lean_mark_persistent(l_Lean_Elab_Command_instInhabitedStructView___closed__1); +l_Lean_Elab_Command_instInhabitedStructView = _init_l_Lean_Elab_Command_instInhabitedStructView(); +lean_mark_persistent(l_Lean_Elab_Command_instInhabitedStructView); +l_Lean_Elab_Command_instInhabitedStructParentInfo___closed__1 = _init_l_Lean_Elab_Command_instInhabitedStructParentInfo___closed__1(); +lean_mark_persistent(l_Lean_Elab_Command_instInhabitedStructParentInfo___closed__1); +l_Lean_Elab_Command_instInhabitedStructParentInfo___closed__2 = _init_l_Lean_Elab_Command_instInhabitedStructParentInfo___closed__2(); +lean_mark_persistent(l_Lean_Elab_Command_instInhabitedStructParentInfo___closed__2); +l_Lean_Elab_Command_instInhabitedStructParentInfo = _init_l_Lean_Elab_Command_instInhabitedStructParentInfo(); +lean_mark_persistent(l_Lean_Elab_Command_instInhabitedStructParentInfo); l_Lean_Elab_Command_StructFieldKind_noConfusion___rarg___closed__1 = _init_l_Lean_Elab_Command_StructFieldKind_noConfusion___rarg___closed__1(); lean_mark_persistent(l_Lean_Elab_Command_StructFieldKind_noConfusion___rarg___closed__1); l_Lean_Elab_Command_instInhabitedStructFieldKind = _init_l_Lean_Elab_Command_instInhabitedStructFieldKind(); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__1 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__1(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__1); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__2 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__2(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__2); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__3 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__3(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__3); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__4 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__4(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__4); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__5 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__5(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__5); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__6 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__6(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__6); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__7 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__7(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__7); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__8 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__8(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__8); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__9 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__9(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__9); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__10 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__10(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__10); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__11 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__11(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__11); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__12 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__12(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__12); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__13 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__13(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__13); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__14 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__14(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__14); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__15 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__15(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__15); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__16 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__16(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__16); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__17 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__17(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__17); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__18 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__18(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__18); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__19 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__19(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__19); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__20 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__20(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__20); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__21 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__21(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__21); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__22 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__22(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__22); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__23 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__23(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__23); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__24 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__24(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__24); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__25 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__25(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__25); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__26 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__26(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__26); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__1 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__1(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__1); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__2 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__2(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__2); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__3 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__3(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__3); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__4 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__4(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__4); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__5 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__5(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__5); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__6 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__6(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__6); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__7 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__7(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__7); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__8 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__8(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__8); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__9 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__9(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__9); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__10 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__10(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__10); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__11 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__11(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__11); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__12 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__12(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__12); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__13 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__13(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__13); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__14 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__14(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__14); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__15 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__15(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__15); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__16 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__16(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__16); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__17 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__17(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__17); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__18 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__18(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__18); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__19 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__19(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__19); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__20 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__20(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__20); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__21 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__21(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__21); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__22 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__22(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__22); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__23 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__23(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__23); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__24 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__24(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__24); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__25 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__25(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__25); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__26 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__26(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_481____closed__26); l_Lean_Elab_Command_instReprStructFieldKind___closed__1 = _init_l_Lean_Elab_Command_instReprStructFieldKind___closed__1(); lean_mark_persistent(l_Lean_Elab_Command_instReprStructFieldKind___closed__1); l_Lean_Elab_Command_instReprStructFieldKind = _init_l_Lean_Elab_Command_instReprStructFieldKind(); lean_mark_persistent(l_Lean_Elab_Command_instReprStructFieldKind); l_Lean_Elab_Command_instInhabitedStructFieldInfo___closed__1 = _init_l_Lean_Elab_Command_instInhabitedStructFieldInfo___closed__1(); lean_mark_persistent(l_Lean_Elab_Command_instInhabitedStructFieldInfo___closed__1); -l_Lean_Elab_Command_instInhabitedStructFieldInfo___closed__2 = _init_l_Lean_Elab_Command_instInhabitedStructFieldInfo___closed__2(); -lean_mark_persistent(l_Lean_Elab_Command_instInhabitedStructFieldInfo___closed__2); l_Lean_Elab_Command_instInhabitedStructFieldInfo = _init_l_Lean_Elab_Command_instInhabitedStructFieldInfo(); lean_mark_persistent(l_Lean_Elab_Command_instInhabitedStructFieldInfo); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__1 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__1(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__1); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__2 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__2(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__2); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__3 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__3(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__3); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__4 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__4(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__4); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__5 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__5(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__5); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__6 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__6(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__6); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__7 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__7(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__7); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__8 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__8(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__8); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__9 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__9(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__9); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__10 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__10(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__10); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__11 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__11(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__11); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__12 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__12(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__12); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__13 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__13(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__13); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__14 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__14(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__14); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__15 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__15(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__15); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__16 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__16(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__16); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__17 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__17(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__17); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__18 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__18(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__18); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__19 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__19(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__19); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__20 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__20(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__20); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__21 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__21(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__21); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__22 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__22(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__22); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__23 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__23(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__23); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__24 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__24(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__24); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__25 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__25(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__25); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__1 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__1(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__1); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__2 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__2(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__2); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__3 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__3(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__3); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__4 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__4(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__4); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__5 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__5(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__5); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__6 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__6(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__6); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__7 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__7(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__7); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__8 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__8(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__8); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__9 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__9(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__9); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__10 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__10(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__10); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__11 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__11(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__11); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__12 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__12(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__12); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__13 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__13(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__13); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__14 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__14(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__14); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__15 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__15(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__15); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__16 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__16(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__16); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__17 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__17(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__17); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__18 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__18(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__18); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__19 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__19(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__19); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__20 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__20(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__20); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__21 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__21(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__21); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__22 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__22(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__22); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__23 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__23(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__23); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__24 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__24(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__24); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__25 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__25(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__25); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__26 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__26(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__26); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__27 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__27(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__27); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__28 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__28(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_698____closed__28); l_Lean_Elab_Command_instReprStructFieldInfo___closed__1 = _init_l_Lean_Elab_Command_instReprStructFieldInfo___closed__1(); lean_mark_persistent(l_Lean_Elab_Command_instReprStructFieldInfo___closed__1); l_Lean_Elab_Command_instReprStructFieldInfo = _init_l_Lean_Elab_Command_instReprStructFieldInfo(); lean_mark_persistent(l_Lean_Elab_Command_instReprStructFieldInfo); +l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__1 = _init_l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__1(); +lean_mark_persistent(l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__1); +l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__2 = _init_l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__2(); +lean_mark_persistent(l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__2); +l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__3 = _init_l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__3(); +lean_mark_persistent(l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__3); +l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__4 = _init_l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__4(); +l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__5 = _init_l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__5(); +lean_mark_persistent(l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__5); +l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__6 = _init_l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__6(); +lean_mark_persistent(l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__6); +l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__7 = _init_l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__7(); +lean_mark_persistent(l_Lean_Elab_Command_instInhabitedElabStructHeaderResult___closed__7); +l_Lean_Elab_Command_instInhabitedElabStructHeaderResult = _init_l_Lean_Elab_Command_instInhabitedElabStructHeaderResult(); +lean_mark_persistent(l_Lean_Elab_Command_instInhabitedElabStructHeaderResult); l___private_Lean_Elab_Structure_0__Lean_Elab_Command_defaultCtorName___closed__1 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_defaultCtorName___closed__1(); lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_defaultCtorName___closed__1); l___private_Lean_Elab_Structure_0__Lean_Elab_Command_defaultCtorName___closed__2 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_defaultCtorName___closed__2(); lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_defaultCtorName___closed__2); l___private_Lean_Elab_Structure_0__Lean_Elab_Command_defaultCtorName = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_defaultCtorName(); lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_defaultCtorName); -l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__1 = _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__1(); -lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__1); -l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__2 = _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__2(); -lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__2); -l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__3 = _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__3(); -lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__3); -l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__4 = _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__4(); -lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__4); -l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__5 = _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__5(); -lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__5); -l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__6 = _init_l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__6(); -lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___closed__6); -l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__9___rarg___closed__1 = _init_l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__9___rarg___closed__1(); -lean_mark_persistent(l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__9___rarg___closed__1); -l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__9___rarg___closed__2 = _init_l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__9___rarg___closed__2(); -lean_mark_persistent(l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__9___rarg___closed__2); -l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__1 = _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__1); -l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__2 = _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__2); -l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__3 = _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__3); -l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__4 = _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__4); -l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__5 = _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__5(); -lean_mark_persistent(l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__5); -l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2___closed__1 = _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2___closed__1(); -lean_mark_persistent(l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2___closed__1); -l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2___closed__2 = _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2___closed__2(); -lean_mark_persistent(l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2___closed__2); -l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2___closed__3 = _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2___closed__3(); -lean_mark_persistent(l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2___closed__3); -l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2___closed__4 = _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2___closed__4(); -lean_mark_persistent(l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2___closed__4); -l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__1 = _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__1(); -lean_mark_persistent(l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__1); -l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__2 = _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__2(); -lean_mark_persistent(l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__2); -l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__3 = _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__3(); -lean_mark_persistent(l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__3); -l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__4 = _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__4(); -lean_mark_persistent(l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__4); -l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__5 = _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__5(); -lean_mark_persistent(l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__5); -l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__6 = _init_l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__6(); -lean_mark_persistent(l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__6); -l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1 = _init_l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1(); -lean_mark_persistent(l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1); -l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__1 = _init_l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__1(); -lean_mark_persistent(l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__1); -l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__2 = _init_l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__2(); -lean_mark_persistent(l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__2); -l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__3 = _init_l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__3(); -lean_mark_persistent(l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__3); -l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__4 = _init_l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__4(); -lean_mark_persistent(l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__4); -l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__1 = _init_l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__1(); -lean_mark_persistent(l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__1); -l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__2 = _init_l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__2(); -lean_mark_persistent(l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__2); -l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__3 = _init_l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__3(); -lean_mark_persistent(l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__3); -l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__4 = _init_l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__4(); -lean_mark_persistent(l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__4); -l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__5 = _init_l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__5(); -lean_mark_persistent(l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__5); -l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__6 = _init_l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__6(); -lean_mark_persistent(l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__6); -l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__7 = _init_l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__7(); -lean_mark_persistent(l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__7); -l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___closed__1 = _init_l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___closed__1(); -lean_mark_persistent(l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___closed__1); -l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___closed__2 = _init_l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___closed__2(); -lean_mark_persistent(l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___closed__2); -l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__1___closed__1 = _init_l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__1___closed__1); -l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__1___closed__2 = _init_l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__1___closed__2); -l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__2___closed__1 = _init_l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__2___closed__1(); -lean_mark_persistent(l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__2___closed__1); -l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__2___closed__2 = _init_l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__2___closed__2(); -lean_mark_persistent(l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__2___closed__2); -l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__3___closed__1 = _init_l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__3___closed__1(); -lean_mark_persistent(l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__3___closed__1); -l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__3___closed__2 = _init_l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__3___closed__2(); -lean_mark_persistent(l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__3___closed__2); -l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___closed__1 = _init_l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___closed__1(); -lean_mark_persistent(l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___closed__1); -l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___closed__2 = _init_l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___closed__2(); -lean_mark_persistent(l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___closed__2); -l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__1 = _init_l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__1(); -lean_mark_persistent(l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__1); -l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__2 = _init_l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__2(); -lean_mark_persistent(l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__2); -l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__3 = _init_l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__3(); -lean_mark_persistent(l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__3); -l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__4 = _init_l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__4(); -lean_mark_persistent(l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__4); -l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__5 = _init_l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__5(); -lean_mark_persistent(l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__5); -l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__6 = _init_l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__6(); -lean_mark_persistent(l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__6); -l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__7 = _init_l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__7(); -lean_mark_persistent(l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__7); l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__2___closed__1 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__2___closed__1(); lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__2___closed__1); l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__2___closed__2 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___lambda__2___closed__2(); @@ -35763,8 +34845,6 @@ l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__1 = _i lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__1); l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__2 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__2(); lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__2); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__3 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__3(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__3); l_Lean_Elab_Command_checkValidFieldModifier___lambda__1___closed__1 = _init_l_Lean_Elab_Command_checkValidFieldModifier___lambda__1___closed__1(); lean_mark_persistent(l_Lean_Elab_Command_checkValidFieldModifier___lambda__1___closed__1); l_Lean_Elab_Command_checkValidFieldModifier___lambda__1___closed__2 = _init_l_Lean_Elab_Command_checkValidFieldModifier___lambda__1___closed__2(); @@ -35793,36 +34873,42 @@ l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Comman lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__1); l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__2 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__2(); lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__2); +l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__3 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__3(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__3); +l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__4 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__4(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__4); +l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__5 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__5(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__5); +l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__6 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__6(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__6); +l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__7 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__7(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__7); +l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__8 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__8(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__8); +l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__9 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__9(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__9); +l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__10 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__10(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__10); +l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__11 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__11(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__11); +l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__12 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__12(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__12); +l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__13 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__13(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__13); +l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__14 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__14(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__14); +l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__15 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__15(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__15); +l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__16 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__16(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__16); +l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__17 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__17(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__17); +l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__18 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__18(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__18); l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__1 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__1(); lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__1); l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__2 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__2(); lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__2); -l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__3 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__3(); -lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__3); -l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__4 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__4(); -lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__4); -l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__5 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__5(); -lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__5); -l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__6 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__6(); -lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__6); -l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__7 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__7(); -lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__7); -l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__8 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__8(); -lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__8); -l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__9 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__9(); -lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__9); -l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__10 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__10(); -lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__10); -l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__11 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__11(); -lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__11); -l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__12 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__12(); -lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__12); -l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__13 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__13(); -lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__13); -l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__14 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__14(); -lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__14); -l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__15 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__15(); -lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__15); l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4___closed__1 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4___closed__1(); lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4___closed__1); l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4___closed__2 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4___closed__2(); @@ -35831,22 +34917,18 @@ l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Comman lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__1); l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__2 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__2(); lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__2); -l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__1 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__1(); -lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__1); -l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__2 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__2(); -lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__2); -l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__3 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__3(); -lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__3); -l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__4 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__4(); -lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__4); -l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__5 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__5(); -lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__5); -l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__6 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__6(); -lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__6); -l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__7 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__7(); -lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__7); -l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__8 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__8(); -lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__8); +l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__3 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__3(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__3); +l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__4 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__4(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__4); +l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__5 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__5(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__5); +l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__6 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__6(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__6); +l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__7 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__7(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__7); +l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__8 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__8(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__8); l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__1 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__1(); lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__1); l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__2 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__2(); @@ -35855,23 +34937,13 @@ l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Comman lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__3); l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__4 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__4(); lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__4); -l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__1 = _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__1(); -lean_mark_persistent(l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__1); -l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__2 = _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__2(); -lean_mark_persistent(l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__2); -l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__3 = _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__3(); -lean_mark_persistent(l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__3); -l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__4 = _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__4(); -lean_mark_persistent(l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__4); -l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__5 = _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__5(); -lean_mark_persistent(l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__5); -l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__6 = _init_l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__6(); -lean_mark_persistent(l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__6); l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__1 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__1(); lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__1); l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__2 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__2(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__2); l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__3 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__3(); l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__4 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__4(); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__5 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__5(); l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__1 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__1(); lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__1); l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__2 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__2(); @@ -35912,30 +34984,35 @@ l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__19 = lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__19); l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__20 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__20(); lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__20); +l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_structureSyntaxToView___spec__1___closed__1 = _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_structureSyntaxToView___spec__1___closed__1(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_structureSyntaxToView___spec__1___closed__1); +l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_structureSyntaxToView___spec__1___closed__2 = _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_structureSyntaxToView___spec__1___closed__2(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_structureSyntaxToView___spec__1___closed__2); +l_Lean_Elab_Command_structureSyntaxToView___closed__1 = _init_l_Lean_Elab_Command_structureSyntaxToView___closed__1(); +lean_mark_persistent(l_Lean_Elab_Command_structureSyntaxToView___closed__1); +l_Lean_Elab_Command_structureSyntaxToView___closed__2 = _init_l_Lean_Elab_Command_structureSyntaxToView___closed__2(); +lean_mark_persistent(l_Lean_Elab_Command_structureSyntaxToView___closed__2); +l_Lean_Elab_Command_structureSyntaxToView___closed__3 = _init_l_Lean_Elab_Command_structureSyntaxToView___closed__3(); +lean_mark_persistent(l_Lean_Elab_Command_structureSyntaxToView___closed__3); +l_Lean_Elab_Command_structureSyntaxToView___closed__4 = _init_l_Lean_Elab_Command_structureSyntaxToView___closed__4(); +lean_mark_persistent(l_Lean_Elab_Command_structureSyntaxToView___closed__4); +l_Lean_Elab_Command_structureSyntaxToView___closed__5 = _init_l_Lean_Elab_Command_structureSyntaxToView___closed__5(); +lean_mark_persistent(l_Lean_Elab_Command_structureSyntaxToView___closed__5); +l_Lean_Elab_Command_structureSyntaxToView___closed__6 = _init_l_Lean_Elab_Command_structureSyntaxToView___closed__6(); +lean_mark_persistent(l_Lean_Elab_Command_structureSyntaxToView___closed__6); +l_Lean_Elab_Command_structureSyntaxToView___closed__7 = _init_l_Lean_Elab_Command_structureSyntaxToView___closed__7(); +lean_mark_persistent(l_Lean_Elab_Command_structureSyntaxToView___closed__7); +l_Lean_Elab_Command_structureSyntaxToView___closed__8 = _init_l_Lean_Elab_Command_structureSyntaxToView___closed__8(); +lean_mark_persistent(l_Lean_Elab_Command_structureSyntaxToView___closed__8); +l_Lean_Elab_Command_structureSyntaxToView___closed__9 = _init_l_Lean_Elab_Command_structureSyntaxToView___closed__9(); +lean_mark_persistent(l_Lean_Elab_Command_structureSyntaxToView___closed__9); l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___closed__1 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___closed__1(); lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___closed__1); l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___closed__2 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___closed__2(); lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___closed__2); l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___closed__3 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___closed__3(); lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___closed__3); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__1 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__1(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__1); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__2 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__2(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__2); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__3 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__3(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__3); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__4 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__4(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__4); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__5 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__5(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__5); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__6 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__6(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__6); -if (builtin) {res = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990_(lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -l_Lean_Elab_Command_structureDiamondWarning = lean_io_result_get_value(res); -lean_mark_persistent(l_Lean_Elab_Command_structureDiamondWarning); -lean_dec_ref(res); -}l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__1 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__1(); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__1 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__1(); lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__1); l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__2 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__2(); lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__2); @@ -35953,6 +35030,8 @@ l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___ lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__2); l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3(); lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__4 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__4(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__4); l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__3___closed__1 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__3___closed__1(); lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__3___closed__1); l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___closed__1 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___closed__1(); @@ -36011,8 +35090,8 @@ l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyField lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__8); l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkToParentName___closed__1 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkToParentName___closed__1(); lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkToParentName___closed__1); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___closed__1 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___closed__1(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___closed__1); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg___closed__1 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg___closed__1(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabParents_go___rarg___closed__1); l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabFieldTypeValue___lambda__2___closed__1 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabFieldTypeValue___lambda__2___closed__1(); lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabFieldTypeValue___lambda__2___closed__1); l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4___closed__1 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4___closed__1(); @@ -36083,12 +35162,42 @@ l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields_go___spec__2___closed__9); l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields_go___spec__2___closed__10 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields_go___spec__2___closed__10(); lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields_go___spec__2___closed__10); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__1 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__1(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__1); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__2 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__2(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__2); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__3 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__3(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__3); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__4 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__4(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__4); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__5 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__5(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__5); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__6 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__6(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__6); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__7 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__7(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___lambda__2___closed__7); l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___closed__1 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___closed__1(); lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___closed__1); l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___closed__2 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___closed__2(); lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse___closed__2); l___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectLevelParamsInStructure___closed__1 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectLevelParamsInStructure___closed__1(); lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectLevelParamsInStructure___closed__1); +l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__1 = _init_l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__1(); +lean_mark_persistent(l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__1); +l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__2 = _init_l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__2(); +lean_mark_persistent(l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__2); +l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__3 = _init_l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__3(); +lean_mark_persistent(l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__3); +l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__4 = _init_l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__4(); +lean_mark_persistent(l_Lean_setEnv___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___spec__5___closed__4); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___closed__1 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___closed__1(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___closed__1); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___closed__2 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___closed__2(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___closed__2); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___closed__3 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___closed__3(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___closed__3); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___closed__4 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___closed__4(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addProjections___closed__4); l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___closed__1 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___closed__1(); lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___closed__1); l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___closed__2 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___closed__2(); @@ -36115,6 +35224,10 @@ l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Comman lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___closed__1); l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___closed__2 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___closed__2(); lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___closed__2); +l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___closed__3 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___closed__3(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___closed__3); +l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___closed__4 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___closed__4(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___closed__4); l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___closed__1 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___closed__1(); lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___closed__1); l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___boxed__const__1 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___boxed__const__1(); @@ -36143,93 +35256,69 @@ l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___ lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___closed__1); l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___closed__2 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___closed__2(); lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___closed__2); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___closed__3 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___closed__3(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___closed__3); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___closed__4 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___closed__4(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___closed__4); -l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__4___closed__1 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__4___closed__1(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__4___closed__1); -l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__4___closed__2 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__4___closed__2(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__4___closed__2); -l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__4___closed__3 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__4___closed__3(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__4___closed__3); -l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__4___closed__4 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__4___closed__4(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__4___closed__4); -l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__11___closed__1 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__11___closed__1(); -lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__11___closed__1); -l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__11___closed__2 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__11___closed__2(); -lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__11___closed__2); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__3___closed__1 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__3___closed__1(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__3___closed__1); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__4___closed__1 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__4___closed__1(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__4___closed__1); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__4___closed__2 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__4___closed__2(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__4___closed__2); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__4___closed__3 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__4___closed__3(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__4___closed__3); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___closed__1 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___closed__1(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___closed__1); -l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___closed__2 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___closed__2(); -lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___closed__2); -l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1___lambda__1___closed__1 = _init_l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1___lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1___lambda__1___closed__1); -l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1___lambda__1___closed__2 = _init_l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1___lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1___lambda__1___closed__2); -l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1___closed__1 = _init_l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1___closed__1(); -lean_mark_persistent(l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1___closed__1); -l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1___closed__2 = _init_l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1___closed__2(); -lean_mark_persistent(l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1___closed__2); -l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___spec__2___closed__1 = _init_l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___spec__2___closed__1(); -lean_mark_persistent(l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___spec__2___closed__1); -l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___spec__2___closed__2 = _init_l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___spec__2___closed__2(); -lean_mark_persistent(l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___spec__2___closed__2); -l_Lean_Elab_Command_elabStructure___closed__1 = _init_l_Lean_Elab_Command_elabStructure___closed__1(); -lean_mark_persistent(l_Lean_Elab_Command_elabStructure___closed__1); -l_Lean_Elab_Command_elabStructure___closed__2 = _init_l_Lean_Elab_Command_elabStructure___closed__2(); -lean_mark_persistent(l_Lean_Elab_Command_elabStructure___closed__2); -l_Lean_Elab_Command_elabStructure___closed__3 = _init_l_Lean_Elab_Command_elabStructure___closed__3(); -lean_mark_persistent(l_Lean_Elab_Command_elabStructure___closed__3); -l_Lean_Elab_Command_elabStructure___closed__4 = _init_l_Lean_Elab_Command_elabStructure___closed__4(); -lean_mark_persistent(l_Lean_Elab_Command_elabStructure___closed__4); -l_Lean_Elab_Command_elabStructure___closed__5 = _init_l_Lean_Elab_Command_elabStructure___closed__5(); -lean_mark_persistent(l_Lean_Elab_Command_elabStructure___closed__5); -l_Lean_Elab_Command_elabStructure___closed__6 = _init_l_Lean_Elab_Command_elabStructure___closed__6(); -lean_mark_persistent(l_Lean_Elab_Command_elabStructure___closed__6); -l_Lean_Elab_Command_elabStructure___closed__7 = _init_l_Lean_Elab_Command_elabStructure___closed__7(); -lean_mark_persistent(l_Lean_Elab_Command_elabStructure___closed__7); -l_Lean_Elab_Command_elabStructure___closed__8 = _init_l_Lean_Elab_Command_elabStructure___closed__8(); -lean_mark_persistent(l_Lean_Elab_Command_elabStructure___closed__8); -l_Lean_Elab_Command_elabStructure___closed__9 = _init_l_Lean_Elab_Command_elabStructure___closed__9(); -lean_mark_persistent(l_Lean_Elab_Command_elabStructure___closed__9); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__1 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__1(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__1); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__2 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__2(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__2); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__3 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__3(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__3); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__4 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__4(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__4); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__5 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__5(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__5); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__6 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__6(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__6); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__7 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__7(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__7); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__8 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__8(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__8); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__9 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__9(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__9); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__10 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__10(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__10); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__11 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__11(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__11); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__12 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__12(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__12); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__13 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__13(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__13); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__14 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__14(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__14); -if (builtin) {res = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022_(lean_io_mk_world()); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__1 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__1(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__1); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__2 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__2(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__2); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__3 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__3(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__3); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__4 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__4(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__4); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__5 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__5(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__5); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__6 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__6(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__3___closed__6); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__5___closed__1 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__5___closed__1(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__5___closed__1); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__5___closed__2 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__5___closed__2(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructHeader___lambda__5___closed__2); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkInductiveType___lambda__3___closed__1 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkInductiveType___lambda__3___closed__1(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkInductiveType___lambda__3___closed__1); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkInductiveType___lambda__3___closed__2 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkInductiveType___lambda__3___closed__2(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkInductiveType___lambda__3___closed__2); +l_Lean_Elab_Command_mkStructureDecl___lambda__3___closed__1 = _init_l_Lean_Elab_Command_mkStructureDecl___lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Elab_Command_mkStructureDecl___lambda__3___closed__1); +l_Lean_Elab_Command_mkStructureDecl___lambda__5___closed__1 = _init_l_Lean_Elab_Command_mkStructureDecl___lambda__5___closed__1(); +lean_mark_persistent(l_Lean_Elab_Command_mkStructureDecl___lambda__5___closed__1); +l_Lean_Elab_Command_mkStructureDecl___lambda__5___closed__2 = _init_l_Lean_Elab_Command_mkStructureDecl___lambda__5___closed__2(); +lean_mark_persistent(l_Lean_Elab_Command_mkStructureDecl___lambda__5___closed__2); +l_Lean_Elab_Command_mkStructureDecl___lambda__8___closed__1 = _init_l_Lean_Elab_Command_mkStructureDecl___lambda__8___closed__1(); +lean_mark_persistent(l_Lean_Elab_Command_mkStructureDecl___lambda__8___closed__1); +l_Lean_Elab_Command_mkStructureDecl___lambda__8___closed__2 = _init_l_Lean_Elab_Command_mkStructureDecl___lambda__8___closed__2(); +lean_mark_persistent(l_Lean_Elab_Command_mkStructureDecl___lambda__8___closed__2); +l_Lean_Elab_Command_elabStructure___lambda__2___closed__1 = _init_l_Lean_Elab_Command_elabStructure___lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Elab_Command_elabStructure___lambda__2___closed__1); +l_Lean_Elab_Command_elabStructure___lambda__2___closed__2 = _init_l_Lean_Elab_Command_elabStructure___lambda__2___closed__2(); +lean_mark_persistent(l_Lean_Elab_Command_elabStructure___lambda__2___closed__2); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__1 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__1(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__1); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__2 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__2(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__2); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__3 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__3(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__3); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__4 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__4(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__4); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__5 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__5(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__5); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__6 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__6(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__6); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__7 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__7(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__7); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__8 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__8(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__8); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__9 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__9(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__9); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__10 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__10(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__10); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__11 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__11(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__11); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__12 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__12(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__12); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__13 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__13(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__13); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__14 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__14(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311____closed__14); +if (builtin) {res = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_15311_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }return lean_io_result_mk_ok(lean_box(0)); diff --git a/stage0/stdlib/Lean/Elab/Syntax.c b/stage0/stdlib/Lean/Elab/Syntax.c index dfd6f9fe28d6..335e51d1bff0 100644 --- a/stage0/stdlib/Lean/Elab/Syntax.c +++ b/stage0/stdlib/Lean/Elab/Syntax.c @@ -413,7 +413,6 @@ static lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyn static lean_object* l_Lean_Elab_Command_checkRuleKind___closed__2; lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); lean_object* l_Lean_Syntax_node3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Term_toParserDescr_processSeq___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabSyntax___lambda__7___closed__3; static lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__61; lean_object* l_Lean_Name_append(lean_object*, lean_object*); @@ -518,7 +517,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_toParserDescr_processSepBy___lambda__1 static lean_object* l_Lean_Elab_Command_elabSyntax___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_toParserDescr_processAlias___lambda__2(lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); -lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Environment_contains(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__17; extern lean_object* l_Lean_inheritedTraceOptions; @@ -612,6 +610,7 @@ uint8_t lean_uint32_dec_eq(uint32_t, uint32_t); static lean_object* l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__19; static lean_object* l_Lean_Elab_Term_toParserDescr_processNonReserved___closed__11; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_toParserDescr_processAlias___spec__6___lambda__1___closed__11; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Term_toParserDescr_processSeq___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); lean_object* l_Lean_isTracingEnabledFor___at_Lean_Elab_Command_runLinters___spec__11(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Term_checkLeftRec___spec__7___closed__4; @@ -633,6 +632,7 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_mkName lean_object* l_Lean_Syntax_node1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_toParserDescr_processSeq___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_toParserDescr_process___closed__7; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Term_toParserDescr_processSeq___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__66; static lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__43; static lean_object* l_Lean_Elab_Command_elabSyntax___lambda__4___closed__15; @@ -660,7 +660,6 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclareSyntaxCat_d lean_object* l_Array_mkArray1___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_resolveSyntaxKind___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Term_elabParserName___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Term_toParserDescr_processSeq___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandNoKindMacroRulesAux___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__12; static lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__44; @@ -770,6 +769,7 @@ uint8_t lean_usize_dec_lt(size_t, size_t); static lean_object* l_Lean_Elab_checkSyntaxNodeKind___at_Lean_Elab_Command_resolveSyntaxKind___spec__2___closed__1; static lean_object* l_Lean_Elab_Command_elabSyntax___lambda__4___closed__5; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabSyntax__1(lean_object*); +lean_object* l_Lean_throwError___at_Lean_withSetOptionIn___spec__7(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__4; static lean_object* l_Lean_Elab_Term_toParserDescr_process___closed__13; static lean_object* l_Lean_Elab_Term_toParserDescr_processNonReserved___closed__10; @@ -12040,7 +12040,7 @@ return x_84; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Term_toParserDescr_processSeq___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Term_toParserDescr_processSeq___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { lean_object* x_16; uint8_t x_17; @@ -12406,7 +12406,7 @@ lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -x_20 = l_Array_mapIdxM_map___at_Lean_Elab_Term_toParserDescr_processSeq___spec__1(x_11, x_11, x_18, x_12, lean_box(0), x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_17); +x_20 = l_Array_mapFinIdxM_map___at_Lean_Elab_Term_toParserDescr_processSeq___spec__1(x_11, x_11, x_18, x_12, lean_box(0), x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_17); lean_dec(x_11); if (lean_obj_tag(x_20) == 0) { @@ -12822,11 +12822,11 @@ lean_dec(x_1); return x_11; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Term_toParserDescr_processSeq___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Term_toParserDescr_processSeq___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { lean_object* x_16; -x_16 = l_Array_mapIdxM_map___at_Lean_Elab_Term_toParserDescr_processSeq___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +x_16 = l_Array_mapFinIdxM_map___at_Lean_Elab_Term_toParserDescr_processSeq___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); lean_dec(x_7); lean_dec(x_2); lean_dec(x_1); @@ -19904,7 +19904,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_expandDeclId___spec__4(x_2, x_3, x_4, x_8); +x_12 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__7(x_2, x_3, x_4, x_8); return x_12; } else @@ -19942,7 +19942,7 @@ lean_ctor_set(x_23, 7, x_19); lean_ctor_set(x_23, 8, x_20); lean_ctor_set(x_23, 9, x_21); lean_ctor_set_uint8(x_23, sizeof(void*)*10, x_22); -x_24 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_2, x_23, x_4, x_8); +x_24 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__7(x_2, x_23, x_4, x_8); return x_24; } } diff --git a/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/Reflect.c b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/Reflect.c index e1dfa7d5ed41..175865630f64 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/Reflect.c +++ b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/Reflect.c @@ -45,6 +45,7 @@ static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lam lean_object* l_Lean_mkAppB(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_isTracingEnabledFor___at_Lean_Elab_Tactic_BVDecide_Frontend_M_lookup___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__5; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__28; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_M_lookup___closed__7; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go(lean_object*, lean_object*); size_t lean_uint64_to_usize(uint64_t); @@ -70,6 +71,7 @@ static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBoolExpr_go__ static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__3; lean_object* lean_array_fget(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_M_atoms___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__26; lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_M_atomsAssignment___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_panic___at_Lean_Elab_Tactic_BVDecide_Frontend_M_lookup___spec__9___closed__1; @@ -291,6 +293,7 @@ static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprGate___closed static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprGate___lambda__1___closed__4; uint8_t lean_nat_dec_le(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__27; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_M_lookup___closed__4; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVUnOp___lambda__1___closed__13; uint8_t lean_usize_dec_lt(size_t, size_t); @@ -309,6 +312,7 @@ static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_M_run___rarg___closed__ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinPred___lambda__1___boxed(lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVPred___closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVUnOp___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__52; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprGate___lambda__1___closed__3; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); lean_object* l___private_Init_Data_Repr_0__Nat_reprFast(lean_object*); @@ -579,6 +583,37 @@ x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__26() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("sdiv", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__27() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__3; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__4; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__26; +x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__28() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__27; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1(uint8_t x_1) { _start: { @@ -619,12 +654,18 @@ lean_object* x_7; x_7 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__22; return x_7; } -default: +case 6: { lean_object* x_8; x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__25; return x_8; } +default: +{ +lean_object* x_9; +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__28; +return x_9; +} } } } @@ -1272,12 +1313,22 @@ return x_3; static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__28() { _start: { +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__27; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__29() { +_start: +{ lean_object* x_1; x_1 = lean_mk_string_unchecked("un", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__29() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__30() { _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; @@ -1285,22 +1336,22 @@ x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___close x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__3; x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__28; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__29; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__30() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__31() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__29; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__30; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__31() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__32() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -1310,7 +1361,7 @@ x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__32() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__33() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -1320,7 +1371,7 @@ x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__33() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__34() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -1330,7 +1381,7 @@ x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__34() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__35() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -1340,7 +1391,7 @@ x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__35() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__36() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -1350,7 +1401,7 @@ x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__36() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__37() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -1360,7 +1411,7 @@ x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__37() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__38() { _start: { lean_object* x_1; @@ -1368,7 +1419,7 @@ x_1 = lean_mk_string_unchecked("append", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__38() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__39() { _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; @@ -1376,22 +1427,22 @@ x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___close x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__3; x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__37; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__38; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__39() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___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_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__38; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__39; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__40() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__41() { _start: { lean_object* x_1; @@ -1399,7 +1450,7 @@ x_1 = lean_mk_string_unchecked("replicate", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__41() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__42() { _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; @@ -1407,22 +1458,22 @@ x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___close x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__3; x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__40; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__41; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__42() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___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_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__41; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__42; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__43() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__44() { _start: { lean_object* x_1; @@ -1430,7 +1481,7 @@ x_1 = lean_mk_string_unchecked("signExtend", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__44() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__45() { _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; @@ -1438,22 +1489,22 @@ x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___close x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__3; x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__43; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__44; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__45() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__46() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__44; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__45; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__46() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__47() { _start: { lean_object* x_1; @@ -1461,7 +1512,7 @@ x_1 = lean_mk_string_unchecked("shiftLeft", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__47() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__48() { _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; @@ -1469,22 +1520,22 @@ x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___close x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__3; x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__46; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__47; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__48() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__49() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__47; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__48; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__49() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__50() { _start: { lean_object* x_1; @@ -1492,7 +1543,7 @@ x_1 = lean_mk_string_unchecked("shiftRight", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__50() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__51() { _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; @@ -1500,17 +1551,17 @@ x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___close x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__3; x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__49; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__50; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__51() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__52() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__50; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__51; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } @@ -1644,7 +1695,7 @@ x_53 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__26; x_54 = l_Lean_mkApp4(x_52, x_34, x_35, x_53, x_36); return x_54; } -default: +case 6: { lean_object* x_55; lean_object* x_56; lean_object* x_57; x_55 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__20; @@ -1652,192 +1703,200 @@ x_56 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__27; x_57 = l_Lean_mkApp4(x_55, x_34, x_35, x_56, x_36); return x_57; } +default: +{ +lean_object* x_58; lean_object* x_59; lean_object* x_60; +x_58 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__20; +x_59 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__28; +x_60 = l_Lean_mkApp4(x_58, x_34, x_35, x_59, x_36); +return x_60; +} } } case 5: { -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); +lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; +x_61 = lean_ctor_get(x_2, 1); +lean_inc(x_61); +x_62 = lean_ctor_get(x_2, 2); +lean_inc(x_62); lean_dec(x_2); lean_inc(x_1); -x_60 = l_Lean_mkNatLit(x_1); -x_61 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go(x_1, x_59); -switch (lean_obj_tag(x_58)) { +x_63 = l_Lean_mkNatLit(x_1); +x_64 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go(x_1, x_62); +switch (lean_obj_tag(x_61)) { case 0: { -lean_object* x_62; lean_object* x_63; lean_object* x_64; -x_62 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__30; -x_63 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__31; -x_64 = l_Lean_mkApp3(x_62, x_60, x_63, x_61); -return x_64; +lean_object* x_65; lean_object* x_66; lean_object* x_67; +x_65 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__31; +x_66 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__32; +x_67 = l_Lean_mkApp3(x_65, x_63, x_66, x_64); +return x_67; } case 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; -x_65 = lean_ctor_get(x_58, 0); -lean_inc(x_65); -lean_dec(x_58); -x_66 = l_Lean_mkNatLit(x_65); -x_67 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__32; -x_68 = l_Lean_Expr_app___override(x_67, x_66); -x_69 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__30; -x_70 = l_Lean_mkApp3(x_69, x_60, x_68, x_61); -return x_70; +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_68 = lean_ctor_get(x_61, 0); +lean_inc(x_68); +lean_dec(x_61); +x_69 = l_Lean_mkNatLit(x_68); +x_70 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__33; +x_71 = l_Lean_Expr_app___override(x_70, x_69); +x_72 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__31; +x_73 = l_Lean_mkApp3(x_72, x_63, x_71, x_64); +return x_73; } case 2: { -lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; -x_71 = lean_ctor_get(x_58, 0); -lean_inc(x_71); -lean_dec(x_58); -x_72 = l_Lean_mkNatLit(x_71); -x_73 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__33; -x_74 = l_Lean_Expr_app___override(x_73, x_72); -x_75 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__30; -x_76 = l_Lean_mkApp3(x_75, x_60, x_74, x_61); -return x_76; +lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; +x_74 = lean_ctor_get(x_61, 0); +lean_inc(x_74); +lean_dec(x_61); +x_75 = l_Lean_mkNatLit(x_74); +x_76 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__34; +x_77 = l_Lean_Expr_app___override(x_76, x_75); +x_78 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__31; +x_79 = l_Lean_mkApp3(x_78, x_63, x_77, x_64); +return x_79; } case 3: { -lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; -x_77 = lean_ctor_get(x_58, 0); -lean_inc(x_77); -lean_dec(x_58); -x_78 = l_Lean_mkNatLit(x_77); -x_79 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__34; -x_80 = l_Lean_Expr_app___override(x_79, x_78); -x_81 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__30; -x_82 = l_Lean_mkApp3(x_81, x_60, x_80, x_61); -return x_82; +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_80 = lean_ctor_get(x_61, 0); +lean_inc(x_80); +lean_dec(x_61); +x_81 = l_Lean_mkNatLit(x_80); +x_82 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__35; +x_83 = l_Lean_Expr_app___override(x_82, x_81); +x_84 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__31; +x_85 = l_Lean_mkApp3(x_84, x_63, x_83, x_64); +return x_85; } case 4: { -lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; -x_83 = lean_ctor_get(x_58, 0); -lean_inc(x_83); -lean_dec(x_58); -x_84 = l_Lean_mkNatLit(x_83); -x_85 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__35; -x_86 = l_Lean_Expr_app___override(x_85, x_84); -x_87 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__30; -x_88 = l_Lean_mkApp3(x_87, x_60, x_86, x_61); -return x_88; +lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; +x_86 = lean_ctor_get(x_61, 0); +lean_inc(x_86); +lean_dec(x_61); +x_87 = l_Lean_mkNatLit(x_86); +x_88 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__36; +x_89 = l_Lean_Expr_app___override(x_88, x_87); +x_90 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__31; +x_91 = l_Lean_mkApp3(x_90, x_63, x_89, x_64); +return x_91; } default: { -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_58, 0); -lean_inc(x_89); -lean_dec(x_58); -x_90 = l_Lean_mkNatLit(x_89); -x_91 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__36; -x_92 = l_Lean_Expr_app___override(x_91, x_90); -x_93 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__30; -x_94 = l_Lean_mkApp3(x_93, x_60, x_92, x_61); -return x_94; +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_92 = lean_ctor_get(x_61, 0); +lean_inc(x_92); +lean_dec(x_61); +x_93 = l_Lean_mkNatLit(x_92); +x_94 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__37; +x_95 = l_Lean_Expr_app___override(x_94, x_93); +x_96 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__31; +x_97 = l_Lean_mkApp3(x_96, x_63, x_95, x_64); +return x_97; } } } case 6: { -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_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_dec(x_1); -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_ctor_get(x_2, 2); -lean_inc(x_97); -x_98 = lean_ctor_get(x_2, 3); +x_98 = lean_ctor_get(x_2, 0); lean_inc(x_98); +x_99 = lean_ctor_get(x_2, 1); +lean_inc(x_99); +x_100 = lean_ctor_get(x_2, 2); +lean_inc(x_100); +x_101 = lean_ctor_get(x_2, 3); +lean_inc(x_101); lean_dec(x_2); -lean_inc(x_95); -x_99 = l_Lean_mkNatLit(x_95); -lean_inc(x_96); -x_100 = l_Lean_mkNatLit(x_96); -x_101 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go(x_95, x_97); -x_102 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go(x_96, x_98); -x_103 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__39; -x_104 = l_Lean_mkApp4(x_103, x_99, x_100, x_101, x_102); -return x_104; +lean_inc(x_98); +x_102 = l_Lean_mkNatLit(x_98); +lean_inc(x_99); +x_103 = l_Lean_mkNatLit(x_99); +x_104 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go(x_98, x_100); +x_105 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go(x_99, x_101); +x_106 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__40; +x_107 = l_Lean_mkApp4(x_106, x_102, x_103, x_104, x_105); +return x_107; } case 7: { -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_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_1); -x_105 = lean_ctor_get(x_2, 0); -lean_inc(x_105); -x_106 = lean_ctor_get(x_2, 1); -lean_inc(x_106); -x_107 = lean_ctor_get(x_2, 2); -lean_inc(x_107); +x_108 = lean_ctor_get(x_2, 0); +lean_inc(x_108); +x_109 = lean_ctor_get(x_2, 1); +lean_inc(x_109); +x_110 = lean_ctor_get(x_2, 2); +lean_inc(x_110); lean_dec(x_2); -lean_inc(x_105); -x_108 = l_Lean_mkNatLit(x_105); -x_109 = l_Lean_mkNatLit(x_106); -x_110 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go(x_105, x_107); -x_111 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__42; -x_112 = l_Lean_mkApp3(x_111, x_108, x_109, x_110); -return x_112; +lean_inc(x_108); +x_111 = l_Lean_mkNatLit(x_108); +x_112 = l_Lean_mkNatLit(x_109); +x_113 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go(x_108, x_110); +x_114 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__43; +x_115 = l_Lean_mkApp3(x_114, x_111, x_112, x_113); +return x_115; } case 8: { -lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; -x_113 = lean_ctor_get(x_2, 0); -lean_inc(x_113); -x_114 = lean_ctor_get(x_2, 2); -lean_inc(x_114); +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 = lean_ctor_get(x_2, 0); +lean_inc(x_116); +x_117 = lean_ctor_get(x_2, 2); +lean_inc(x_117); lean_dec(x_2); -lean_inc(x_113); -x_115 = l_Lean_mkNatLit(x_113); -x_116 = l_Lean_mkNatLit(x_1); -x_117 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go(x_113, x_114); -x_118 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__45; -x_119 = l_Lean_mkApp3(x_118, x_115, x_116, x_117); -return x_119; +lean_inc(x_116); +x_118 = l_Lean_mkNatLit(x_116); +x_119 = l_Lean_mkNatLit(x_1); +x_120 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go(x_116, x_117); +x_121 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__46; +x_122 = l_Lean_mkApp3(x_121, x_118, x_119, x_120); +return x_122; } case 9: { -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_120 = lean_ctor_get(x_2, 1); -lean_inc(x_120); -x_121 = lean_ctor_get(x_2, 2); -lean_inc(x_121); -x_122 = lean_ctor_get(x_2, 3); -lean_inc(x_122); +lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; +x_123 = lean_ctor_get(x_2, 1); +lean_inc(x_123); +x_124 = lean_ctor_get(x_2, 2); +lean_inc(x_124); +x_125 = lean_ctor_get(x_2, 3); +lean_inc(x_125); lean_dec(x_2); lean_inc(x_1); -x_123 = l_Lean_mkNatLit(x_1); -lean_inc(x_120); -x_124 = l_Lean_mkNatLit(x_120); -x_125 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go(x_1, x_121); -x_126 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go(x_120, x_122); -x_127 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__48; -x_128 = l_Lean_mkApp4(x_127, x_123, x_124, x_125, x_126); -return x_128; +x_126 = l_Lean_mkNatLit(x_1); +lean_inc(x_123); +x_127 = l_Lean_mkNatLit(x_123); +x_128 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go(x_1, x_124); +x_129 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go(x_123, x_125); +x_130 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__49; +x_131 = l_Lean_mkApp4(x_130, x_126, x_127, x_128, x_129); +return x_131; } default: { -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_129 = lean_ctor_get(x_2, 1); -lean_inc(x_129); -x_130 = lean_ctor_get(x_2, 2); -lean_inc(x_130); -x_131 = lean_ctor_get(x_2, 3); -lean_inc(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; +x_132 = lean_ctor_get(x_2, 1); +lean_inc(x_132); +x_133 = lean_ctor_get(x_2, 2); +lean_inc(x_133); +x_134 = lean_ctor_get(x_2, 3); +lean_inc(x_134); lean_dec(x_2); lean_inc(x_1); -x_132 = l_Lean_mkNatLit(x_1); -lean_inc(x_129); -x_133 = l_Lean_mkNatLit(x_129); -x_134 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go(x_1, x_130); -x_135 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go(x_129, x_131); -x_136 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__51; -x_137 = l_Lean_mkApp4(x_136, x_132, x_133, x_134, x_135); -return x_137; +x_135 = l_Lean_mkNatLit(x_1); +lean_inc(x_132); +x_136 = l_Lean_mkNatLit(x_132); +x_137 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go(x_1, x_133); +x_138 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go(x_132, x_134); +x_139 = l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__52; +x_140 = l_Lean_mkApp4(x_139, x_135, x_136, x_137, x_138); +return x_140; } } } @@ -4820,7 +4879,7 @@ static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_M_lookup___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_Elab_Tactic_BVDecide_Frontend_M_lookup___closed__9; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_M_lookup___closed__10; -x_3 = lean_unsigned_to_nat(155u); +x_3 = lean_unsigned_to_nat(156u); x_4 = lean_unsigned_to_nat(6u); x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_M_lookup___closed__11; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -5580,6 +5639,12 @@ l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__24 lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__24); l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__25 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__25(); lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__25); +l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__26 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__26(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__26); +l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__27 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__27(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__27); +l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__28 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__28(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___lambda__1___closed__28); l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___closed__1(); lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___closed__1); l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVBinOp___closed__2(); @@ -5740,6 +5805,8 @@ l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__50 = _init_l_ lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__50); l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__51 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__51(); lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__51); +l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__52 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__52(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr_go___closed__52); l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr___closed__1(); lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr___closed__1); l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBVExpr___closed__2(); diff --git a/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/ReifiedBVExpr.c b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/ReifiedBVExpr.c index 1f75fc0e3efa..5ede596ea5ca 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/ReifiedBVExpr.c +++ b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/ReifiedBVExpr.c @@ -13,307 +13,321 @@ #ifdef __cplusplus extern "C" { #endif -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__10; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__11___closed__2; lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__28___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__31(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_unaryReflection___closed__6; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__6; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__20; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__13; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__1; lean_object* l_Lean_mkNatLit(lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__6; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__24; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__3(lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__4; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__31___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__1; lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_M_lookup(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__6; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__51; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__60; lean_object* l_Lean_Meta_getNatValue_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_getNatOrBvValue_x3f___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__26___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__45; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__34; LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_getNatOrBvValue_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__14; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__18; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkApp8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__8; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__1; lean_object* l_Lean_mkAppB(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__13; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__4; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_getNatOrBvValue_x3f___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__27; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__4; uint8_t l_Lean_Expr_isApp(lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__10; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__58; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__40; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__22; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__1(lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__5; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__29(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__12; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_unaryReflection___closed__7; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__10; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__17; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__19; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__23___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__8; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__30___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__3(lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__48; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__7; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__24(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftConstLikeReflection(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__32; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__21(lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__38; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__32___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__50; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__33; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goBvLit___closed__4; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__26; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__5; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__20; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__14; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goBvLit___closed__5; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__17; lean_object* l_Lean_Name_mkStr5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__4; lean_object* l_Lean_Expr_cleanupAnnotations(lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__31; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__24___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__5___closed__1; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__19; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__53; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_unaryReflection___closed__8; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__44; lean_object* l_Lean_mkApp4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__29___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goBvLit(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__9; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__15(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__17(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__25(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__4; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__5; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__57; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__24___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__5; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__7; lean_object* l_Lean_Level_ofNat(lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__8; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__5___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__46; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__29(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_getNatOrBvValue_x3f___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__9; uint8_t l_Lean_Expr_hasMVar(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__47; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__5; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__39; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__32(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkApp6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_getNatOrBvValue_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__25___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__1; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_unaryReflection___closed__4; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__28___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__5; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___closed__3; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__30; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__29___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_rotateReflection___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__56; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_rotateReflection___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__1; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__30(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__36; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__33; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__26___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__5; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__14; lean_object* lean_st_ref_take(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__25(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_getNatOrBvValue_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__43; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__39; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__7; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__28(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__23; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__25___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__7; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__21(lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__27___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__9___closed__2; lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_M_atomsAssignment(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__9; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___closed__1; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__26___closed__1; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goBvLit___closed__1; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__1; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_unaryReflection___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__15; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__31(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__23; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__9___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__31; lean_object* l_Lean_Meta_getBitVecValue_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__5; lean_object* l_Lean_Expr_appArg(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goBvLit___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__21; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__7; lean_object* lean_st_ref_get(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__25; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__24(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__26; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__24___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__25___closed__2; lean_object* l_Lean_Expr_appFnCleanup(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__7; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__31___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__9; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__20(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__54; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__55; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__3; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__37; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__19; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__30; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__8; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__7; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__30(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__6; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__9___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__23(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__38; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__22; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__3; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__8; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__7___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__27; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__15; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__10; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__8; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_getNatOrBvValue_x3f___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__41; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__25; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11___closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_unaryReflection___closed__11; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__24___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__7; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__32; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__6; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__28___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__49; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__50; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__23(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__27___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__20; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__21; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__29; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__5; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__10; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__6; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__27(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__6; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goBvLit___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__7___closed__1; lean_object* l_Lean_Name_mkStr6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__5; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__28(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__28; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__3; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__5; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__4; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__6; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__41; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__25___closed__1; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__9; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__17(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__3; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_unaryReflection___closed__10; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_app___override(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__42; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__18(lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__29; uint8_t lean_nat_dec_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_getNatOrBvValue_x3f___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkApp3(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__32___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__26(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__23; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__23___closed__1; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__6; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__28; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__16; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__2; lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__32(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__35; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__27; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofOrAtom(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__15; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__26; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__37; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__11; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__3; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__5; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__27___closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__25; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__12; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__12; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isConstOf(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__13; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_unaryReflection___closed__9; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__5___closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__24; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__30___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__23___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__11; lean_object* lean_nat_mul(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__22; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__28___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__61; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__7; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; lean_object* l_Lean_Meta_instantiateMVarsIfMVarApp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__52; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__7; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__44; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__7___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__31___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__23___closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__5; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftConstReflection(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__49; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftConstReflection(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__8; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__1(lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_unaryReflection___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__43; lean_object* l_Lean_instantiateMVarsCore(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__35; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_unaryReflection(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__11___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__9; +LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__9; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__9; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__21; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__18; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_getNatOrBvValue_x3f___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__24; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__29___closed__1; LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__30___closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__46; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__6; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__47; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__10; lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_rotateReflection(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__27(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__29___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_rotateReflection(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_unaryCongrProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__34; -LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__26(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__4; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__8; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__16; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__9___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__26___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__45; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__42; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__63; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__16; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__36; lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__15(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__20(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__62; lean_object* lean_nat_add(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_unaryReflection___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_getNatOrBvValue_x3f___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__2; lean_object* l_Lean_mkApp5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__4; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__51; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__18(lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__18; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__5___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__48; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__5; -LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__27___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__4; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__59; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__11; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goBvLit___closed__6; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__10; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__40; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__30___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__17; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryCongrProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; lean_object* l_Lean_Meta_whnfR(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_unaryReflection___closed__3; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__3; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__6; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__7___closed__1; +LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1() { _start: @@ -1016,7 +1030,7 @@ lean_dec(x_1); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { uint8_t x_8; @@ -1123,7 +1137,7 @@ return x_35; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; @@ -1322,7 +1336,7 @@ return x_44; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; @@ -1353,7 +1367,7 @@ lean_inc(x_12); x_13 = lean_ctor_get(x_11, 1); lean_inc(x_13); lean_dec(x_11); -x_14 = l_Lean_instantiateMVars___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom___spec__1(x_12, x_2, x_3, x_4, x_5, x_6, x_13); +x_14 = l_Lean_instantiateMVars___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom___spec__1(x_12, x_2, x_3, x_4, x_5, x_6, x_13); x_15 = lean_ctor_get(x_14, 0); lean_inc(x_15); x_16 = lean_ctor_get(x_14, 1); @@ -1391,7 +1405,7 @@ return x_27; else { lean_object* x_28; -x_28 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom___lambda__1(x_1, x_22, x_2, x_3, x_4, x_5, x_6, x_16); +x_28 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom___lambda__1(x_1, x_22, x_2, x_3, x_4, x_5, x_6, x_16); lean_dec(x_22); return x_28; } @@ -1456,11 +1470,11 @@ return x_36; } } } -LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; -x_8 = l_Lean_instantiateMVars___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Lean_instantiateMVars___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); @@ -1469,11 +1483,11 @@ lean_dec(x_2); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; -x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_2); return x_9; } @@ -1558,7 +1572,7 @@ lean_object* x_10; lean_object* x_11; x_10 = lean_ctor_get(x_8, 1); lean_inc(x_10); lean_dec(x_8); -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_2, x_3, x_4, x_5, x_6, x_10); +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom(x_1, x_2, x_3, x_4, x_5, x_6, x_10); if (lean_obj_tag(x_11) == 0) { uint8_t x_12; @@ -2092,122 +2106,7 @@ return x_29; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofOrAtom(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_2); -lean_inc(x_1); -x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -if (lean_obj_tag(x_8) == 0) -{ -lean_object* x_9; -x_9 = lean_ctor_get(x_8, 0); -lean_inc(x_9); -if (lean_obj_tag(x_9) == 0) -{ -lean_object* x_10; lean_object* x_11; -x_10 = lean_ctor_get(x_8, 1); -lean_inc(x_10); -lean_dec(x_8); -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_2, x_3, x_4, x_5, x_6, x_10); -return x_11; -} -else -{ -uint8_t x_12; -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_12 = !lean_is_exclusive(x_8); -if (x_12 == 0) -{ -lean_object* x_13; uint8_t x_14; -x_13 = lean_ctor_get(x_8, 0); -lean_dec(x_13); -x_14 = !lean_is_exclusive(x_9); -if (x_14 == 0) -{ -return x_8; -} -else -{ -lean_object* x_15; lean_object* x_16; -x_15 = lean_ctor_get(x_9, 0); -lean_inc(x_15); -lean_dec(x_9); -x_16 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_16, 0, x_15); -lean_ctor_set(x_8, 0, x_16); -return x_8; -} -} -else -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_17 = lean_ctor_get(x_8, 1); -lean_inc(x_17); -lean_dec(x_8); -x_18 = lean_ctor_get(x_9, 0); -lean_inc(x_18); -if (lean_is_exclusive(x_9)) { - lean_ctor_release(x_9, 0); - x_19 = x_9; -} else { - lean_dec_ref(x_9); - x_19 = lean_box(0); -} -if (lean_is_scalar(x_19)) { - x_20 = lean_alloc_ctor(1, 1, 0); -} else { - x_20 = x_19; -} -lean_ctor_set(x_20, 0, x_18); -x_21 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_21, 0, x_20); -lean_ctor_set(x_21, 1, x_17); -return x_21; -} -} -} -else -{ -uint8_t x_22; -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_22 = !lean_is_exclusive(x_8); -if (x_22 == 0) -{ -return x_8; -} -else -{ -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_8, 0); -x_24 = lean_ctor_get(x_8, 1); -lean_inc(x_24); -lean_inc(x_23); -lean_dec(x_8); -x_25 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_25, 0, x_23); -lean_ctor_set(x_25, 1, x_24); -return x_25; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__1(lean_object* x_1) { _start: { lean_object* x_2; @@ -2216,7 +2115,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__1() { _start: { lean_object* x_1; @@ -2224,7 +2123,7 @@ x_1 = lean_mk_string_unchecked("BVUnOp", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__2() { _start: { lean_object* x_1; @@ -2232,20 +2131,20 @@ x_1 = lean_mk_string_unchecked("rotateRight", 11, 11); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__2; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__2; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4() { _start: { lean_object* x_1; @@ -2253,7 +2152,7 @@ x_1 = lean_mk_string_unchecked("Reflect", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__5() { _start: { lean_object* x_1; @@ -2261,40 +2160,40 @@ x_1 = lean_mk_string_unchecked("rotateRight_congr", 17, 17); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__6() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__5; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__5; x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); return x_7; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__7() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__7() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__1), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__1), 1, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__7; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__3; -x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__6; -x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_rotateReflection(x_1, x_3, x_2, x_10, x_11, x_12, x_4, x_5, x_6, x_7, x_8, x_9); -return x_13; +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__7; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__3; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__6; +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_rotateReflection(x_2, x_1, x_9, x_10, x_11, x_3, x_4, x_5, x_6, x_7, x_8); +return x_12; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__3(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__3(lean_object* x_1) { _start: { lean_object* x_2; @@ -2303,7 +2202,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__1() { _start: { lean_object* x_1; @@ -2311,20 +2210,20 @@ x_1 = lean_mk_string_unchecked("rotateLeft", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__1; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__1; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__3() { _start: { lean_object* x_1; @@ -2332,40 +2231,40 @@ x_1 = lean_mk_string_unchecked("rotateLeft_congr", 16, 16); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__3; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__3; x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); return x_7; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__5() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__3), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__3), 1, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__5; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__2; -x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__4; -x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_rotateReflection(x_1, x_3, x_2, x_10, x_11, x_12, x_4, x_5, x_6, x_7, x_8, x_9); -return x_13; +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__5; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__2; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__4; +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_rotateReflection(x_2, x_1, x_9, x_10, x_11, x_3, x_4, x_5, x_6, x_7, x_8); +return x_12; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__5___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__5___closed__1() { _start: { lean_object* x_1; @@ -2373,21 +2272,21 @@ x_1 = lean_mk_string_unchecked("extract_congr", 13, 13); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__5___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__5___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__5___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__5___closed__1; x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { lean_object* x_14; lean_object* x_15; @@ -2403,7 +2302,7 @@ if (x_16 == 0) { lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; x_17 = lean_ctor_get(x_15, 0); -x_18 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__5___closed__2; +x_18 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__5___closed__2; x_19 = l_Lean_Expr_const___override(x_18, x_2); x_20 = l_Lean_mkApp6(x_19, x_3, x_4, x_5, x_6, x_7, x_17); lean_ctor_set(x_15, 0, x_20); @@ -2417,7 +2316,7 @@ x_22 = lean_ctor_get(x_15, 1); lean_inc(x_22); lean_inc(x_21); lean_dec(x_15); -x_23 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__5___closed__2; +x_23 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__5___closed__2; x_24 = l_Lean_Expr_const___override(x_23, x_2); x_25 = l_Lean_mkApp6(x_24, x_3, x_4, x_5, x_6, x_7, x_21); x_26 = lean_alloc_ctor(0, 2, 0); @@ -2456,7 +2355,7 @@ return x_30; } } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__1() { _start: { lean_object* x_1; @@ -2464,7 +2363,7 @@ x_1 = lean_mk_string_unchecked("extract", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; @@ -2472,484 +2371,440 @@ x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__4; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__1; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__2; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__2; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_11; -lean_inc(x_9); +lean_object* x_10; lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -x_11 = l_Lean_Meta_getNatValue_x3f(x_2, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_11) == 0) +lean_inc(x_5); +x_10 = l_Lean_Meta_getNatValue_x3f(x_1, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_10) == 0) { -lean_object* x_12; -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); -if (lean_obj_tag(x_12) == 0) +lean_object* x_11; +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +if (lean_obj_tag(x_11) == 0) { -lean_object* x_13; lean_object* x_14; +uint8_t x_12; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_13 = lean_ctor_get(x_11, 1); -lean_inc(x_13); -lean_dec(x_11); -x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_5, x_6, x_7, x_8, x_9, x_13); -if (lean_obj_tag(x_14) == 0) -{ -uint8_t x_15; -x_15 = !lean_is_exclusive(x_14); -if (x_15 == 0) -{ -return x_14; -} -else -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_14, 0); -x_17 = lean_ctor_get(x_14, 1); -lean_inc(x_17); -lean_inc(x_16); -lean_dec(x_14); -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_16); -lean_ctor_set(x_18, 1, x_17); -return x_18; -} -} -else -{ -uint8_t x_19; -x_19 = !lean_is_exclusive(x_14); -if (x_19 == 0) +lean_dec(x_1); +x_12 = !lean_is_exclusive(x_10); +if (x_12 == 0) { -return x_14; +lean_object* x_13; lean_object* x_14; +x_13 = lean_ctor_get(x_10, 0); +lean_dec(x_13); +x_14 = lean_box(0); +lean_ctor_set(x_10, 0, x_14); +return x_10; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_14, 0); -x_21 = lean_ctor_get(x_14, 1); -lean_inc(x_21); -lean_inc(x_20); -lean_dec(x_14); -x_22 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_22, 0, x_20); -lean_ctor_set(x_22, 1, x_21); -return x_22; -} +lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_15 = lean_ctor_get(x_10, 1); +lean_inc(x_15); +lean_dec(x_10); +x_16 = lean_box(0); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_16); +lean_ctor_set(x_17, 1, x_15); +return x_17; } } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_11, 1); -lean_inc(x_23); +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_10, 1); +lean_inc(x_18); +lean_dec(x_10); +x_19 = lean_ctor_get(x_11, 0); +lean_inc(x_19); lean_dec(x_11); -x_24 = lean_ctor_get(x_12, 0); -lean_inc(x_24); -lean_dec(x_12); -lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -x_25 = l_Lean_Meta_getNatValue_x3f(x_3, x_6, x_7, x_8, x_9, x_23); -if (lean_obj_tag(x_25) == 0) +lean_inc(x_5); +x_20 = l_Lean_Meta_getNatValue_x3f(x_2, x_5, x_6, x_7, x_8, x_18); +if (lean_obj_tag(x_20) == 0) { -lean_object* x_26; -x_26 = lean_ctor_get(x_25, 0); -lean_inc(x_26); -if (lean_obj_tag(x_26) == 0) +lean_object* x_21; +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +if (lean_obj_tag(x_21) == 0) { -lean_object* x_27; lean_object* x_28; -lean_dec(x_24); +uint8_t x_22; +lean_dec(x_19); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_27 = lean_ctor_get(x_25, 1); -lean_inc(x_27); -lean_dec(x_25); -x_28 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_5, x_6, x_7, x_8, x_9, x_27); -if (lean_obj_tag(x_28) == 0) -{ -uint8_t x_29; -x_29 = !lean_is_exclusive(x_28); -if (x_29 == 0) +lean_dec(x_1); +x_22 = !lean_is_exclusive(x_20); +if (x_22 == 0) { -return x_28; +lean_object* x_23; lean_object* x_24; +x_23 = lean_ctor_get(x_20, 0); +lean_dec(x_23); +x_24 = lean_box(0); +lean_ctor_set(x_20, 0, x_24); +return x_20; } else { -lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_30 = lean_ctor_get(x_28, 0); -x_31 = lean_ctor_get(x_28, 1); -lean_inc(x_31); -lean_inc(x_30); -lean_dec(x_28); -x_32 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_32, 0, x_30); -lean_ctor_set(x_32, 1, x_31); -return x_32; +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_20, 1); +lean_inc(x_25); +lean_dec(x_20); +x_26 = lean_box(0); +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_25); +return x_27; } } else { -uint8_t x_33; -x_33 = !lean_is_exclusive(x_28); -if (x_33 == 0) +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_20, 1); +lean_inc(x_28); +lean_dec(x_20); +x_29 = lean_ctor_get(x_21, 0); +lean_inc(x_29); +lean_dec(x_21); +lean_inc(x_3); +x_30 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(x_3, x_4, x_5, x_6, x_7, x_8, x_28); +if (lean_obj_tag(x_30) == 0) { -return x_28; -} -else -{ -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_28, 0); -x_35 = lean_ctor_get(x_28, 1); -lean_inc(x_35); -lean_inc(x_34); -lean_dec(x_28); -x_36 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_36, 0, x_34); -lean_ctor_set(x_36, 1, x_35); -return x_36; -} -} -} -else -{ -lean_object* x_37; lean_object* x_38; lean_object* x_39; -lean_dec(x_1); -x_37 = lean_ctor_get(x_25, 1); -lean_inc(x_37); -lean_dec(x_25); -x_38 = lean_ctor_get(x_26, 0); -lean_inc(x_38); -lean_dec(x_26); -lean_inc(x_4); -x_39 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofOrAtom(x_4, x_5, x_6, x_7, x_8, x_9, x_37); -if (lean_obj_tag(x_39) == 0) -{ -lean_object* x_40; -x_40 = lean_ctor_get(x_39, 0); -lean_inc(x_40); -if (lean_obj_tag(x_40) == 0) +lean_object* x_31; +x_31 = lean_ctor_get(x_30, 0); +lean_inc(x_31); +if (lean_obj_tag(x_31) == 0) { -uint8_t x_41; -lean_dec(x_38); -lean_dec(x_24); -lean_dec(x_4); +uint8_t x_32; +lean_dec(x_29); +lean_dec(x_19); lean_dec(x_3); lean_dec(x_2); -x_41 = !lean_is_exclusive(x_39); -if (x_41 == 0) +lean_dec(x_1); +x_32 = !lean_is_exclusive(x_30); +if (x_32 == 0) { -lean_object* x_42; lean_object* x_43; -x_42 = lean_ctor_get(x_39, 0); -lean_dec(x_42); -x_43 = lean_box(0); -lean_ctor_set(x_39, 0, x_43); -return x_39; +lean_object* x_33; lean_object* x_34; +x_33 = lean_ctor_get(x_30, 0); +lean_dec(x_33); +x_34 = lean_box(0); +lean_ctor_set(x_30, 0, x_34); +return x_30; } else { -lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_44 = lean_ctor_get(x_39, 1); -lean_inc(x_44); -lean_dec(x_39); -x_45 = lean_box(0); -x_46 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_46, 0, x_45); -lean_ctor_set(x_46, 1, x_44); -return x_46; +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_30, 1); +lean_inc(x_35); +lean_dec(x_30); +x_36 = lean_box(0); +x_37 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_37, 0, x_36); +lean_ctor_set(x_37, 1, x_35); +return x_37; } } else { -uint8_t x_47; -x_47 = !lean_is_exclusive(x_40); -if (x_47 == 0) +uint8_t x_38; +x_38 = !lean_is_exclusive(x_31); +if (x_38 == 0) { -uint8_t x_48; -x_48 = !lean_is_exclusive(x_39); -if (x_48 == 0) +uint8_t x_39; +x_39 = !lean_is_exclusive(x_30); +if (x_39 == 0) { -lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; uint8_t x_61; -x_49 = lean_ctor_get(x_40, 0); -x_50 = lean_ctor_get(x_39, 0); -lean_dec(x_50); -x_51 = lean_ctor_get(x_49, 0); -lean_inc(x_51); -x_52 = lean_ctor_get(x_49, 1); -lean_inc(x_52); -x_53 = lean_ctor_get(x_49, 3); -lean_inc(x_53); -lean_inc(x_38); -lean_inc(x_51); -x_54 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_54, 0, x_51); -lean_ctor_set(x_54, 1, x_24); -lean_ctor_set(x_54, 2, x_38); -lean_ctor_set(x_54, 3, x_52); -x_55 = lean_box(0); -lean_inc(x_51); -x_56 = l_Lean_mkNatLit(x_51); -x_57 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__3; -lean_inc(x_53); -lean_inc(x_3); +lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; uint8_t x_52; +x_40 = lean_ctor_get(x_31, 0); +x_41 = lean_ctor_get(x_30, 0); +lean_dec(x_41); +x_42 = lean_ctor_get(x_40, 0); +lean_inc(x_42); +x_43 = lean_ctor_get(x_40, 1); +lean_inc(x_43); +x_44 = lean_ctor_get(x_40, 3); +lean_inc(x_44); +lean_inc(x_29); +lean_inc(x_42); +x_45 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_45, 0, x_42); +lean_ctor_set(x_45, 1, x_19); +lean_ctor_set(x_45, 2, x_29); +lean_ctor_set(x_45, 3, x_43); +x_46 = lean_box(0); +lean_inc(x_42); +x_47 = l_Lean_mkNatLit(x_42); +x_48 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__3; +lean_inc(x_44); lean_inc(x_2); -lean_inc(x_56); -x_58 = l_Lean_mkApp4(x_57, x_56, x_2, x_3, x_53); -x_59 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_59, 0, x_51); -lean_closure_set(x_59, 1, x_53); -lean_inc(x_49); -x_60 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__5), 13, 6); -lean_closure_set(x_60, 0, x_49); -lean_closure_set(x_60, 1, x_55); -lean_closure_set(x_60, 2, x_2); -lean_closure_set(x_60, 3, x_3); -lean_closure_set(x_60, 4, x_56); -lean_closure_set(x_60, 5, x_4); -x_61 = !lean_is_exclusive(x_49); -if (x_61 == 0) -{ -lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_62 = lean_ctor_get(x_49, 3); -lean_dec(x_62); -x_63 = lean_ctor_get(x_49, 2); -lean_dec(x_63); -x_64 = lean_ctor_get(x_49, 1); -lean_dec(x_64); -x_65 = lean_ctor_get(x_49, 0); -lean_dec(x_65); -x_66 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_66, 0, x_59); -lean_closure_set(x_66, 1, x_60); -lean_ctor_set(x_49, 3, x_58); -lean_ctor_set(x_49, 2, x_66); -lean_ctor_set(x_49, 1, x_54); -lean_ctor_set(x_49, 0, x_38); -return x_39; +lean_inc(x_1); +lean_inc(x_47); +x_49 = l_Lean_mkApp4(x_48, x_47, x_1, x_2, x_44); +x_50 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_50, 0, x_42); +lean_closure_set(x_50, 1, x_44); +lean_inc(x_40); +x_51 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__5), 13, 6); +lean_closure_set(x_51, 0, x_40); +lean_closure_set(x_51, 1, x_46); +lean_closure_set(x_51, 2, x_1); +lean_closure_set(x_51, 3, x_2); +lean_closure_set(x_51, 4, x_47); +lean_closure_set(x_51, 5, x_3); +x_52 = !lean_is_exclusive(x_40); +if (x_52 == 0) +{ +lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_53 = lean_ctor_get(x_40, 3); +lean_dec(x_53); +x_54 = lean_ctor_get(x_40, 2); +lean_dec(x_54); +x_55 = lean_ctor_get(x_40, 1); +lean_dec(x_55); +x_56 = lean_ctor_get(x_40, 0); +lean_dec(x_56); +x_57 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_57, 0, x_50); +lean_closure_set(x_57, 1, x_51); +lean_ctor_set(x_40, 3, x_49); +lean_ctor_set(x_40, 2, x_57); +lean_ctor_set(x_40, 1, x_45); +lean_ctor_set(x_40, 0, x_29); +return x_30; } else { -lean_object* x_67; lean_object* x_68; -lean_dec(x_49); -x_67 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_67, 0, x_59); -lean_closure_set(x_67, 1, x_60); -x_68 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_68, 0, x_38); -lean_ctor_set(x_68, 1, x_54); -lean_ctor_set(x_68, 2, x_67); -lean_ctor_set(x_68, 3, x_58); -lean_ctor_set(x_40, 0, x_68); -return x_39; +lean_object* x_58; lean_object* x_59; +lean_dec(x_40); +x_58 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_58, 0, x_50); +lean_closure_set(x_58, 1, x_51); +x_59 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_59, 0, x_29); +lean_ctor_set(x_59, 1, x_45); +lean_ctor_set(x_59, 2, x_58); +lean_ctor_set(x_59, 3, x_49); +lean_ctor_set(x_31, 0, x_59); +return x_30; } } else { -lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; -x_69 = lean_ctor_get(x_40, 0); -x_70 = lean_ctor_get(x_39, 1); -lean_inc(x_70); -lean_dec(x_39); -x_71 = lean_ctor_get(x_69, 0); -lean_inc(x_71); -x_72 = lean_ctor_get(x_69, 1); -lean_inc(x_72); -x_73 = lean_ctor_get(x_69, 3); -lean_inc(x_73); -lean_inc(x_38); -lean_inc(x_71); -x_74 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_74, 0, x_71); -lean_ctor_set(x_74, 1, x_24); -lean_ctor_set(x_74, 2, x_38); -lean_ctor_set(x_74, 3, x_72); -x_75 = lean_box(0); -lean_inc(x_71); -x_76 = l_Lean_mkNatLit(x_71); -x_77 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__3; -lean_inc(x_73); -lean_inc(x_3); +lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; +x_60 = lean_ctor_get(x_31, 0); +x_61 = lean_ctor_get(x_30, 1); +lean_inc(x_61); +lean_dec(x_30); +x_62 = lean_ctor_get(x_60, 0); +lean_inc(x_62); +x_63 = lean_ctor_get(x_60, 1); +lean_inc(x_63); +x_64 = lean_ctor_get(x_60, 3); +lean_inc(x_64); +lean_inc(x_29); +lean_inc(x_62); +x_65 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_65, 0, x_62); +lean_ctor_set(x_65, 1, x_19); +lean_ctor_set(x_65, 2, x_29); +lean_ctor_set(x_65, 3, x_63); +x_66 = lean_box(0); +lean_inc(x_62); +x_67 = l_Lean_mkNatLit(x_62); +x_68 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__3; +lean_inc(x_64); lean_inc(x_2); -lean_inc(x_76); -x_78 = l_Lean_mkApp4(x_77, x_76, x_2, x_3, x_73); -x_79 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_79, 0, x_71); -lean_closure_set(x_79, 1, x_73); -lean_inc(x_69); -x_80 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__5), 13, 6); -lean_closure_set(x_80, 0, x_69); -lean_closure_set(x_80, 1, x_75); -lean_closure_set(x_80, 2, x_2); -lean_closure_set(x_80, 3, x_3); -lean_closure_set(x_80, 4, x_76); -lean_closure_set(x_80, 5, x_4); -if (lean_is_exclusive(x_69)) { - lean_ctor_release(x_69, 0); - lean_ctor_release(x_69, 1); - lean_ctor_release(x_69, 2); - lean_ctor_release(x_69, 3); - x_81 = x_69; +lean_inc(x_1); +lean_inc(x_67); +x_69 = l_Lean_mkApp4(x_68, x_67, x_1, x_2, x_64); +x_70 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_70, 0, x_62); +lean_closure_set(x_70, 1, x_64); +lean_inc(x_60); +x_71 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__5), 13, 6); +lean_closure_set(x_71, 0, x_60); +lean_closure_set(x_71, 1, x_66); +lean_closure_set(x_71, 2, x_1); +lean_closure_set(x_71, 3, x_2); +lean_closure_set(x_71, 4, x_67); +lean_closure_set(x_71, 5, x_3); +if (lean_is_exclusive(x_60)) { + lean_ctor_release(x_60, 0); + lean_ctor_release(x_60, 1); + lean_ctor_release(x_60, 2); + lean_ctor_release(x_60, 3); + x_72 = x_60; } else { - lean_dec_ref(x_69); - x_81 = lean_box(0); + lean_dec_ref(x_60); + x_72 = lean_box(0); } -x_82 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_82, 0, x_79); -lean_closure_set(x_82, 1, x_80); -if (lean_is_scalar(x_81)) { - x_83 = lean_alloc_ctor(0, 4, 0); +x_73 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_73, 0, x_70); +lean_closure_set(x_73, 1, x_71); +if (lean_is_scalar(x_72)) { + x_74 = lean_alloc_ctor(0, 4, 0); } else { - x_83 = x_81; + x_74 = x_72; } -lean_ctor_set(x_83, 0, x_38); -lean_ctor_set(x_83, 1, x_74); -lean_ctor_set(x_83, 2, x_82); -lean_ctor_set(x_83, 3, x_78); -lean_ctor_set(x_40, 0, x_83); -x_84 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_84, 0, x_40); -lean_ctor_set(x_84, 1, x_70); -return x_84; +lean_ctor_set(x_74, 0, x_29); +lean_ctor_set(x_74, 1, x_65); +lean_ctor_set(x_74, 2, x_73); +lean_ctor_set(x_74, 3, x_69); +lean_ctor_set(x_31, 0, x_74); +x_75 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_75, 0, x_31); +lean_ctor_set(x_75, 1, x_61); +return x_75; } } else { -lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; -x_85 = lean_ctor_get(x_40, 0); -lean_inc(x_85); -lean_dec(x_40); -x_86 = lean_ctor_get(x_39, 1); -lean_inc(x_86); -if (lean_is_exclusive(x_39)) { - lean_ctor_release(x_39, 0); - lean_ctor_release(x_39, 1); - x_87 = x_39; +lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; +x_76 = lean_ctor_get(x_31, 0); +lean_inc(x_76); +lean_dec(x_31); +x_77 = lean_ctor_get(x_30, 1); +lean_inc(x_77); +if (lean_is_exclusive(x_30)) { + lean_ctor_release(x_30, 0); + lean_ctor_release(x_30, 1); + x_78 = x_30; } else { - lean_dec_ref(x_39); - x_87 = lean_box(0); + lean_dec_ref(x_30); + x_78 = lean_box(0); } -x_88 = lean_ctor_get(x_85, 0); -lean_inc(x_88); -x_89 = lean_ctor_get(x_85, 1); -lean_inc(x_89); -x_90 = lean_ctor_get(x_85, 3); -lean_inc(x_90); -lean_inc(x_38); -lean_inc(x_88); -x_91 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_91, 0, x_88); -lean_ctor_set(x_91, 1, x_24); -lean_ctor_set(x_91, 2, x_38); -lean_ctor_set(x_91, 3, x_89); -x_92 = lean_box(0); -lean_inc(x_88); -x_93 = l_Lean_mkNatLit(x_88); -x_94 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__3; -lean_inc(x_90); -lean_inc(x_3); +x_79 = lean_ctor_get(x_76, 0); +lean_inc(x_79); +x_80 = lean_ctor_get(x_76, 1); +lean_inc(x_80); +x_81 = lean_ctor_get(x_76, 3); +lean_inc(x_81); +lean_inc(x_29); +lean_inc(x_79); +x_82 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_82, 0, x_79); +lean_ctor_set(x_82, 1, x_19); +lean_ctor_set(x_82, 2, x_29); +lean_ctor_set(x_82, 3, x_80); +x_83 = lean_box(0); +lean_inc(x_79); +x_84 = l_Lean_mkNatLit(x_79); +x_85 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__3; +lean_inc(x_81); lean_inc(x_2); -lean_inc(x_93); -x_95 = l_Lean_mkApp4(x_94, x_93, x_2, x_3, x_90); -x_96 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_96, 0, x_88); -lean_closure_set(x_96, 1, x_90); -lean_inc(x_85); -x_97 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__5), 13, 6); -lean_closure_set(x_97, 0, x_85); -lean_closure_set(x_97, 1, x_92); -lean_closure_set(x_97, 2, x_2); -lean_closure_set(x_97, 3, x_3); -lean_closure_set(x_97, 4, x_93); -lean_closure_set(x_97, 5, x_4); -if (lean_is_exclusive(x_85)) { - lean_ctor_release(x_85, 0); - lean_ctor_release(x_85, 1); - lean_ctor_release(x_85, 2); - lean_ctor_release(x_85, 3); - x_98 = x_85; +lean_inc(x_1); +lean_inc(x_84); +x_86 = l_Lean_mkApp4(x_85, x_84, x_1, x_2, x_81); +x_87 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_87, 0, x_79); +lean_closure_set(x_87, 1, x_81); +lean_inc(x_76); +x_88 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__5), 13, 6); +lean_closure_set(x_88, 0, x_76); +lean_closure_set(x_88, 1, x_83); +lean_closure_set(x_88, 2, x_1); +lean_closure_set(x_88, 3, x_2); +lean_closure_set(x_88, 4, x_84); +lean_closure_set(x_88, 5, x_3); +if (lean_is_exclusive(x_76)) { + lean_ctor_release(x_76, 0); + lean_ctor_release(x_76, 1); + lean_ctor_release(x_76, 2); + lean_ctor_release(x_76, 3); + x_89 = x_76; } else { - lean_dec_ref(x_85); - x_98 = lean_box(0); -} -x_99 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_99, 0, x_96); -lean_closure_set(x_99, 1, x_97); -if (lean_is_scalar(x_98)) { - x_100 = lean_alloc_ctor(0, 4, 0); + lean_dec_ref(x_76); + x_89 = lean_box(0); +} +x_90 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_90, 0, x_87); +lean_closure_set(x_90, 1, x_88); +if (lean_is_scalar(x_89)) { + x_91 = lean_alloc_ctor(0, 4, 0); } else { - x_100 = x_98; -} -lean_ctor_set(x_100, 0, x_38); -lean_ctor_set(x_100, 1, x_91); -lean_ctor_set(x_100, 2, x_99); -lean_ctor_set(x_100, 3, x_95); -x_101 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_101, 0, x_100); -if (lean_is_scalar(x_87)) { - x_102 = lean_alloc_ctor(0, 2, 0); + x_91 = x_89; +} +lean_ctor_set(x_91, 0, x_29); +lean_ctor_set(x_91, 1, x_82); +lean_ctor_set(x_91, 2, x_90); +lean_ctor_set(x_91, 3, x_86); +x_92 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_92, 0, x_91); +if (lean_is_scalar(x_78)) { + x_93 = lean_alloc_ctor(0, 2, 0); } else { - x_102 = x_87; + x_93 = x_78; } -lean_ctor_set(x_102, 0, x_101); -lean_ctor_set(x_102, 1, x_86); -return x_102; +lean_ctor_set(x_93, 0, x_92); +lean_ctor_set(x_93, 1, x_77); +return x_93; } } } else { -uint8_t x_103; -lean_dec(x_38); -lean_dec(x_24); -lean_dec(x_4); +uint8_t x_94; +lean_dec(x_29); +lean_dec(x_19); lean_dec(x_3); lean_dec(x_2); -x_103 = !lean_is_exclusive(x_39); -if (x_103 == 0) +lean_dec(x_1); +x_94 = !lean_is_exclusive(x_30); +if (x_94 == 0) { -return x_39; +return x_30; } else { -lean_object* x_104; lean_object* x_105; lean_object* x_106; -x_104 = lean_ctor_get(x_39, 0); -x_105 = lean_ctor_get(x_39, 1); -lean_inc(x_105); -lean_inc(x_104); -lean_dec(x_39); -x_106 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_106, 0, x_104); -lean_ctor_set(x_106, 1, x_105); -return x_106; +lean_object* x_95; lean_object* x_96; lean_object* x_97; +x_95 = lean_ctor_get(x_30, 0); +x_96 = lean_ctor_get(x_30, 1); +lean_inc(x_96); +lean_inc(x_95); +lean_dec(x_30); +x_97 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_97, 0, x_95); +lean_ctor_set(x_97, 1, x_96); +return x_97; } } } } else { -uint8_t x_107; -lean_dec(x_24); -lean_dec(x_9); +uint8_t x_98; +lean_dec(x_19); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -2958,31 +2813,30 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_107 = !lean_is_exclusive(x_25); -if (x_107 == 0) +x_98 = !lean_is_exclusive(x_20); +if (x_98 == 0) { -return x_25; +return x_20; } else { -lean_object* x_108; lean_object* x_109; lean_object* x_110; -x_108 = lean_ctor_get(x_25, 0); -x_109 = lean_ctor_get(x_25, 1); -lean_inc(x_109); -lean_inc(x_108); -lean_dec(x_25); -x_110 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_110, 0, x_108); -lean_ctor_set(x_110, 1, x_109); -return x_110; +lean_object* x_99; lean_object* x_100; lean_object* x_101; +x_99 = lean_ctor_get(x_20, 0); +x_100 = lean_ctor_get(x_20, 1); +lean_inc(x_100); +lean_inc(x_99); +lean_dec(x_20); +x_101 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_101, 0, x_99); +lean_ctor_set(x_101, 1, x_100); +return x_101; } } } } else { -uint8_t x_111; -lean_dec(x_9); +uint8_t x_102; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -2991,28 +2845,28 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_111 = !lean_is_exclusive(x_11); -if (x_111 == 0) +x_102 = !lean_is_exclusive(x_10); +if (x_102 == 0) { -return x_11; +return x_10; } else { -lean_object* x_112; lean_object* x_113; lean_object* x_114; -x_112 = lean_ctor_get(x_11, 0); -x_113 = lean_ctor_get(x_11, 1); -lean_inc(x_113); -lean_inc(x_112); -lean_dec(x_11); -x_114 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_114, 0, x_112); -lean_ctor_set(x_114, 1, x_113); -return x_114; +lean_object* x_103; lean_object* x_104; lean_object* x_105; +x_103 = lean_ctor_get(x_10, 0); +x_104 = lean_ctor_get(x_10, 1); +lean_inc(x_104); +lean_inc(x_103); +lean_dec(x_10); +x_105 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_105, 0, x_103); +lean_ctor_set(x_105, 1, x_104); +return x_105; } } } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__7___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__7___closed__1() { _start: { lean_object* x_1; @@ -3020,21 +2874,21 @@ x_1 = lean_mk_string_unchecked("replicate_congr", 15, 15); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__7___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__7___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__7___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__7___closed__1; x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; @@ -3050,7 +2904,7 @@ if (x_15 == 0) { lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; x_16 = lean_ctor_get(x_14, 0); -x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__7___closed__2; +x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__7___closed__2; x_18 = l_Lean_Expr_const___override(x_17, x_2); x_19 = l_Lean_mkApp5(x_18, x_3, x_4, x_5, x_6, x_16); lean_ctor_set(x_14, 0, x_19); @@ -3064,7 +2918,7 @@ x_21 = lean_ctor_get(x_14, 1); lean_inc(x_21); lean_inc(x_20); lean_dec(x_14); -x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__7___closed__2; +x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__7___closed__2; x_23 = l_Lean_Expr_const___override(x_22, x_2); x_24 = l_Lean_mkApp5(x_23, x_3, x_4, x_5, x_6, x_20); x_25 = lean_alloc_ctor(0, 2, 0); @@ -3102,7 +2956,7 @@ return x_29; } } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__1() { _start: { lean_object* x_1; @@ -3110,7 +2964,7 @@ x_1 = lean_mk_string_unchecked("replicate", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; @@ -3118,460 +2972,413 @@ x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__4; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__1; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__2; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__2; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_10; -lean_inc(x_8); +lean_object* x_9; lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -lean_inc(x_3); -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofOrAtom(x_3, x_4, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_10) == 0) +lean_inc(x_2); +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(x_2, x_3, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_9) == 0) { -lean_object* x_11; -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -if (lean_obj_tag(x_11) == 0) +lean_object* x_10; +x_10 = lean_ctor_get(x_9, 0); +lean_inc(x_10); +if (lean_obj_tag(x_10) == 0) { -uint8_t x_12; -lean_dec(x_8); +uint8_t x_11; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_12 = !lean_is_exclusive(x_10); -if (x_12 == 0) +lean_dec(x_2); +x_11 = !lean_is_exclusive(x_9); +if (x_11 == 0) { -lean_object* x_13; lean_object* x_14; -x_13 = lean_ctor_get(x_10, 0); -lean_dec(x_13); -x_14 = lean_box(0); -lean_ctor_set(x_10, 0, x_14); -return x_10; +lean_object* x_12; lean_object* x_13; +x_12 = lean_ctor_get(x_9, 0); +lean_dec(x_12); +x_13 = lean_box(0); +lean_ctor_set(x_9, 0, x_13); +return x_9; } else { -lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = lean_ctor_get(x_10, 1); -lean_inc(x_15); -lean_dec(x_10); -x_16 = lean_box(0); -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_16); -lean_ctor_set(x_17, 1, x_15); -return x_17; +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_9, 1); +lean_inc(x_14); +lean_dec(x_9); +x_15 = lean_box(0); +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_16, 1, x_14); +return x_16; } } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_10, 1); +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_9, 1); +lean_inc(x_17); +lean_dec(x_9); +x_18 = lean_ctor_get(x_10, 0); lean_inc(x_18); lean_dec(x_10); -x_19 = lean_ctor_get(x_11, 0); -lean_inc(x_19); -lean_dec(x_11); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -x_20 = l_Lean_Meta_getNatValue_x3f(x_2, x_5, x_6, x_7, x_8, x_18); +x_19 = l_Lean_Meta_getNatValue_x3f(x_1, x_4, x_5, x_6, x_7, x_17); +if (lean_obj_tag(x_19) == 0) +{ +lean_object* x_20; +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); if (lean_obj_tag(x_20) == 0) { -lean_object* x_21; -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -if (lean_obj_tag(x_21) == 0) +uint8_t x_21; +lean_dec(x_18); +lean_dec(x_2); +x_21 = !lean_is_exclusive(x_19); +if (x_21 == 0) { lean_object* x_22; lean_object* x_23; -lean_dec(x_19); -lean_dec(x_3); -x_22 = lean_ctor_get(x_20, 1); -lean_inc(x_22); -lean_dec(x_20); -x_23 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_4, x_5, x_6, x_7, x_8, x_22); -if (lean_obj_tag(x_23) == 0) -{ -uint8_t x_24; -x_24 = !lean_is_exclusive(x_23); -if (x_24 == 0) -{ -return x_23; +x_22 = lean_ctor_get(x_19, 0); +lean_dec(x_22); +x_23 = lean_box(0); +lean_ctor_set(x_19, 0, x_23); +return x_19; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_23, 0); -x_26 = lean_ctor_get(x_23, 1); -lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_23); -x_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_26); -return x_27; +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_19, 1); +lean_inc(x_24); +lean_dec(x_19); +x_25 = lean_box(0); +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_24); +return x_26; } } else { -uint8_t x_28; -x_28 = !lean_is_exclusive(x_23); -if (x_28 == 0) +uint8_t x_27; +x_27 = !lean_is_exclusive(x_19); +if (x_27 == 0) { -return x_23; -} -else +lean_object* x_28; uint8_t x_29; +x_28 = lean_ctor_get(x_19, 0); +lean_dec(x_28); +x_29 = !lean_is_exclusive(x_20); +if (x_29 == 0) { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_23, 0); -x_30 = lean_ctor_get(x_23, 1); +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; +x_30 = lean_ctor_get(x_20, 0); +x_31 = lean_ctor_get(x_18, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_18, 1); +lean_inc(x_32); +x_33 = lean_ctor_get(x_18, 3); +lean_inc(x_33); lean_inc(x_30); -lean_inc(x_29); -lean_dec(x_23); -x_31 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_31, 0, x_29); -lean_ctor_set(x_31, 1, x_30); -return x_31; -} -} -} -else -{ -uint8_t x_32; -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_1); -x_32 = !lean_is_exclusive(x_20); -if (x_32 == 0) -{ -lean_object* x_33; uint8_t x_34; -x_33 = lean_ctor_get(x_20, 0); -lean_dec(x_33); -x_34 = !lean_is_exclusive(x_21); -if (x_34 == 0) -{ -lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; -x_35 = lean_ctor_get(x_21, 0); -x_36 = lean_ctor_get(x_19, 0); -lean_inc(x_36); -x_37 = lean_ctor_get(x_19, 1); +lean_inc(x_31); +x_34 = lean_alloc_ctor(7, 3, 0); +lean_ctor_set(x_34, 0, x_31); +lean_ctor_set(x_34, 1, x_30); +lean_ctor_set(x_34, 2, x_32); +x_35 = lean_box(0); +lean_inc(x_31); +x_36 = l_Lean_mkNatLit(x_31); +lean_inc(x_30); +x_37 = l_Lean_mkNatLit(x_30); +x_38 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__3; +lean_inc(x_33); lean_inc(x_37); -x_38 = lean_ctor_get(x_19, 3); -lean_inc(x_38); -lean_inc(x_35); lean_inc(x_36); -x_39 = lean_alloc_ctor(7, 3, 0); -lean_ctor_set(x_39, 0, x_36); -lean_ctor_set(x_39, 1, x_35); -lean_ctor_set(x_39, 2, x_37); -x_40 = lean_box(0); -lean_inc(x_36); -x_41 = l_Lean_mkNatLit(x_36); -lean_inc(x_35); -x_42 = l_Lean_mkNatLit(x_35); -x_43 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__3; -lean_inc(x_38); -lean_inc(x_42); -lean_inc(x_41); -x_44 = l_Lean_mkApp3(x_43, x_41, x_42, x_38); -lean_inc(x_36); -x_45 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_45, 0, x_36); -lean_closure_set(x_45, 1, x_38); -lean_inc(x_19); -x_46 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__7), 12, 5); -lean_closure_set(x_46, 0, x_19); -lean_closure_set(x_46, 1, x_40); -lean_closure_set(x_46, 2, x_42); -lean_closure_set(x_46, 3, x_41); -lean_closure_set(x_46, 4, x_3); -x_47 = !lean_is_exclusive(x_19); -if (x_47 == 0) -{ -lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; -x_48 = lean_ctor_get(x_19, 3); -lean_dec(x_48); -x_49 = lean_ctor_get(x_19, 2); -lean_dec(x_49); -x_50 = lean_ctor_get(x_19, 1); -lean_dec(x_50); -x_51 = lean_ctor_get(x_19, 0); -lean_dec(x_51); -x_52 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_52, 0, x_45); -lean_closure_set(x_52, 1, x_46); -x_53 = lean_nat_mul(x_36, x_35); -lean_dec(x_35); -lean_dec(x_36); -lean_ctor_set(x_19, 3, x_44); -lean_ctor_set(x_19, 2, x_52); -lean_ctor_set(x_19, 1, x_39); -lean_ctor_set(x_19, 0, x_53); -lean_ctor_set(x_21, 0, x_19); -return x_20; +x_39 = l_Lean_mkApp3(x_38, x_36, x_37, x_33); +lean_inc(x_31); +x_40 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_40, 0, x_31); +lean_closure_set(x_40, 1, x_33); +lean_inc(x_18); +x_41 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__7), 12, 5); +lean_closure_set(x_41, 0, x_18); +lean_closure_set(x_41, 1, x_35); +lean_closure_set(x_41, 2, x_37); +lean_closure_set(x_41, 3, x_36); +lean_closure_set(x_41, 4, x_2); +x_42 = !lean_is_exclusive(x_18); +if (x_42 == 0) +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_43 = lean_ctor_get(x_18, 3); +lean_dec(x_43); +x_44 = lean_ctor_get(x_18, 2); +lean_dec(x_44); +x_45 = lean_ctor_get(x_18, 1); +lean_dec(x_45); +x_46 = lean_ctor_get(x_18, 0); +lean_dec(x_46); +x_47 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_47, 0, x_40); +lean_closure_set(x_47, 1, x_41); +x_48 = lean_nat_mul(x_31, x_30); +lean_dec(x_30); +lean_dec(x_31); +lean_ctor_set(x_18, 3, x_39); +lean_ctor_set(x_18, 2, x_47); +lean_ctor_set(x_18, 1, x_34); +lean_ctor_set(x_18, 0, x_48); +lean_ctor_set(x_20, 0, x_18); +return x_19; } else { -lean_object* x_54; lean_object* x_55; lean_object* x_56; -lean_dec(x_19); -x_54 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_54, 0, x_45); -lean_closure_set(x_54, 1, x_46); -x_55 = lean_nat_mul(x_36, x_35); -lean_dec(x_35); -lean_dec(x_36); -x_56 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_56, 0, x_55); -lean_ctor_set(x_56, 1, x_39); -lean_ctor_set(x_56, 2, x_54); -lean_ctor_set(x_56, 3, x_44); -lean_ctor_set(x_21, 0, x_56); -return x_20; +lean_object* x_49; lean_object* x_50; lean_object* x_51; +lean_dec(x_18); +x_49 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_49, 0, x_40); +lean_closure_set(x_49, 1, x_41); +x_50 = lean_nat_mul(x_31, x_30); +lean_dec(x_30); +lean_dec(x_31); +x_51 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_51, 0, x_50); +lean_ctor_set(x_51, 1, x_34); +lean_ctor_set(x_51, 2, x_49); +lean_ctor_set(x_51, 3, x_39); +lean_ctor_set(x_20, 0, x_51); +return x_19; } } else { -lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_57 = lean_ctor_get(x_21, 0); -lean_inc(x_57); -lean_dec(x_21); -x_58 = lean_ctor_get(x_19, 0); -lean_inc(x_58); -x_59 = lean_ctor_get(x_19, 1); +lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; +x_52 = lean_ctor_get(x_20, 0); +lean_inc(x_52); +lean_dec(x_20); +x_53 = lean_ctor_get(x_18, 0); +lean_inc(x_53); +x_54 = lean_ctor_get(x_18, 1); +lean_inc(x_54); +x_55 = lean_ctor_get(x_18, 3); +lean_inc(x_55); +lean_inc(x_52); +lean_inc(x_53); +x_56 = lean_alloc_ctor(7, 3, 0); +lean_ctor_set(x_56, 0, x_53); +lean_ctor_set(x_56, 1, x_52); +lean_ctor_set(x_56, 2, x_54); +x_57 = lean_box(0); +lean_inc(x_53); +x_58 = l_Lean_mkNatLit(x_53); +lean_inc(x_52); +x_59 = l_Lean_mkNatLit(x_52); +x_60 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__3; +lean_inc(x_55); lean_inc(x_59); -x_60 = lean_ctor_get(x_19, 3); -lean_inc(x_60); -lean_inc(x_57); -lean_inc(x_58); -x_61 = lean_alloc_ctor(7, 3, 0); -lean_ctor_set(x_61, 0, x_58); -lean_ctor_set(x_61, 1, x_57); -lean_ctor_set(x_61, 2, x_59); -x_62 = lean_box(0); lean_inc(x_58); -x_63 = l_Lean_mkNatLit(x_58); -lean_inc(x_57); -x_64 = l_Lean_mkNatLit(x_57); -x_65 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__3; -lean_inc(x_60); -lean_inc(x_64); -lean_inc(x_63); -x_66 = l_Lean_mkApp3(x_65, x_63, x_64, x_60); -lean_inc(x_58); -x_67 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_67, 0, x_58); -lean_closure_set(x_67, 1, x_60); -lean_inc(x_19); -x_68 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__7), 12, 5); -lean_closure_set(x_68, 0, x_19); -lean_closure_set(x_68, 1, x_62); -lean_closure_set(x_68, 2, x_64); -lean_closure_set(x_68, 3, x_63); -lean_closure_set(x_68, 4, x_3); -if (lean_is_exclusive(x_19)) { - lean_ctor_release(x_19, 0); - lean_ctor_release(x_19, 1); - lean_ctor_release(x_19, 2); - lean_ctor_release(x_19, 3); - x_69 = x_19; +x_61 = l_Lean_mkApp3(x_60, x_58, x_59, x_55); +lean_inc(x_53); +x_62 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_62, 0, x_53); +lean_closure_set(x_62, 1, x_55); +lean_inc(x_18); +x_63 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__7), 12, 5); +lean_closure_set(x_63, 0, x_18); +lean_closure_set(x_63, 1, x_57); +lean_closure_set(x_63, 2, x_59); +lean_closure_set(x_63, 3, x_58); +lean_closure_set(x_63, 4, x_2); +if (lean_is_exclusive(x_18)) { + lean_ctor_release(x_18, 0); + lean_ctor_release(x_18, 1); + lean_ctor_release(x_18, 2); + lean_ctor_release(x_18, 3); + x_64 = x_18; } else { - lean_dec_ref(x_19); - x_69 = lean_box(0); + lean_dec_ref(x_18); + x_64 = lean_box(0); } -x_70 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_70, 0, x_67); -lean_closure_set(x_70, 1, x_68); -x_71 = lean_nat_mul(x_58, x_57); -lean_dec(x_57); -lean_dec(x_58); -if (lean_is_scalar(x_69)) { - x_72 = lean_alloc_ctor(0, 4, 0); +x_65 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_65, 0, x_62); +lean_closure_set(x_65, 1, x_63); +x_66 = lean_nat_mul(x_53, x_52); +lean_dec(x_52); +lean_dec(x_53); +if (lean_is_scalar(x_64)) { + x_67 = lean_alloc_ctor(0, 4, 0); } else { - x_72 = x_69; -} -lean_ctor_set(x_72, 0, x_71); -lean_ctor_set(x_72, 1, x_61); -lean_ctor_set(x_72, 2, x_70); -lean_ctor_set(x_72, 3, x_66); -x_73 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_73, 0, x_72); -lean_ctor_set(x_20, 0, x_73); -return x_20; + x_67 = x_64; +} +lean_ctor_set(x_67, 0, x_66); +lean_ctor_set(x_67, 1, x_56); +lean_ctor_set(x_67, 2, x_65); +lean_ctor_set(x_67, 3, x_61); +x_68 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_68, 0, x_67); +lean_ctor_set(x_19, 0, x_68); +return x_19; } } else { -lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; -x_74 = lean_ctor_get(x_20, 1); -lean_inc(x_74); -lean_dec(x_20); -x_75 = lean_ctor_get(x_21, 0); -lean_inc(x_75); -if (lean_is_exclusive(x_21)) { - lean_ctor_release(x_21, 0); - x_76 = x_21; +lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; +x_69 = lean_ctor_get(x_19, 1); +lean_inc(x_69); +lean_dec(x_19); +x_70 = lean_ctor_get(x_20, 0); +lean_inc(x_70); +if (lean_is_exclusive(x_20)) { + lean_ctor_release(x_20, 0); + x_71 = x_20; } else { - lean_dec_ref(x_21); - x_76 = lean_box(0); + lean_dec_ref(x_20); + x_71 = lean_box(0); } -x_77 = lean_ctor_get(x_19, 0); -lean_inc(x_77); -x_78 = lean_ctor_get(x_19, 1); +x_72 = lean_ctor_get(x_18, 0); +lean_inc(x_72); +x_73 = lean_ctor_get(x_18, 1); +lean_inc(x_73); +x_74 = lean_ctor_get(x_18, 3); +lean_inc(x_74); +lean_inc(x_70); +lean_inc(x_72); +x_75 = lean_alloc_ctor(7, 3, 0); +lean_ctor_set(x_75, 0, x_72); +lean_ctor_set(x_75, 1, x_70); +lean_ctor_set(x_75, 2, x_73); +x_76 = lean_box(0); +lean_inc(x_72); +x_77 = l_Lean_mkNatLit(x_72); +lean_inc(x_70); +x_78 = l_Lean_mkNatLit(x_70); +x_79 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__3; +lean_inc(x_74); lean_inc(x_78); -x_79 = lean_ctor_get(x_19, 3); -lean_inc(x_79); -lean_inc(x_75); -lean_inc(x_77); -x_80 = lean_alloc_ctor(7, 3, 0); -lean_ctor_set(x_80, 0, x_77); -lean_ctor_set(x_80, 1, x_75); -lean_ctor_set(x_80, 2, x_78); -x_81 = lean_box(0); -lean_inc(x_77); -x_82 = l_Lean_mkNatLit(x_77); -lean_inc(x_75); -x_83 = l_Lean_mkNatLit(x_75); -x_84 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__3; -lean_inc(x_79); -lean_inc(x_83); -lean_inc(x_82); -x_85 = l_Lean_mkApp3(x_84, x_82, x_83, x_79); lean_inc(x_77); -x_86 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_86, 0, x_77); -lean_closure_set(x_86, 1, x_79); -lean_inc(x_19); -x_87 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__7), 12, 5); -lean_closure_set(x_87, 0, x_19); -lean_closure_set(x_87, 1, x_81); -lean_closure_set(x_87, 2, x_83); -lean_closure_set(x_87, 3, x_82); -lean_closure_set(x_87, 4, x_3); -if (lean_is_exclusive(x_19)) { - lean_ctor_release(x_19, 0); - lean_ctor_release(x_19, 1); - lean_ctor_release(x_19, 2); - lean_ctor_release(x_19, 3); - x_88 = x_19; +x_80 = l_Lean_mkApp3(x_79, x_77, x_78, x_74); +lean_inc(x_72); +x_81 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_81, 0, x_72); +lean_closure_set(x_81, 1, x_74); +lean_inc(x_18); +x_82 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__7), 12, 5); +lean_closure_set(x_82, 0, x_18); +lean_closure_set(x_82, 1, x_76); +lean_closure_set(x_82, 2, x_78); +lean_closure_set(x_82, 3, x_77); +lean_closure_set(x_82, 4, x_2); +if (lean_is_exclusive(x_18)) { + lean_ctor_release(x_18, 0); + lean_ctor_release(x_18, 1); + lean_ctor_release(x_18, 2); + lean_ctor_release(x_18, 3); + x_83 = x_18; } else { - lean_dec_ref(x_19); - x_88 = lean_box(0); + lean_dec_ref(x_18); + x_83 = lean_box(0); } -x_89 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_89, 0, x_86); -lean_closure_set(x_89, 1, x_87); -x_90 = lean_nat_mul(x_77, x_75); -lean_dec(x_75); -lean_dec(x_77); -if (lean_is_scalar(x_88)) { - x_91 = lean_alloc_ctor(0, 4, 0); +x_84 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_84, 0, x_81); +lean_closure_set(x_84, 1, x_82); +x_85 = lean_nat_mul(x_72, x_70); +lean_dec(x_70); +lean_dec(x_72); +if (lean_is_scalar(x_83)) { + x_86 = lean_alloc_ctor(0, 4, 0); } else { - x_91 = x_88; -} -lean_ctor_set(x_91, 0, x_90); -lean_ctor_set(x_91, 1, x_80); -lean_ctor_set(x_91, 2, x_89); -lean_ctor_set(x_91, 3, x_85); -if (lean_is_scalar(x_76)) { - x_92 = lean_alloc_ctor(1, 1, 0); + x_86 = x_83; +} +lean_ctor_set(x_86, 0, x_85); +lean_ctor_set(x_86, 1, x_75); +lean_ctor_set(x_86, 2, x_84); +lean_ctor_set(x_86, 3, x_80); +if (lean_is_scalar(x_71)) { + x_87 = lean_alloc_ctor(1, 1, 0); } else { - x_92 = x_76; + x_87 = x_71; } -lean_ctor_set(x_92, 0, x_91); -x_93 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_93, 0, x_92); -lean_ctor_set(x_93, 1, x_74); -return x_93; +lean_ctor_set(x_87, 0, x_86); +x_88 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_88, 0, x_87); +lean_ctor_set(x_88, 1, x_69); +return x_88; } } } else { -uint8_t x_94; -lean_dec(x_19); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_94 = !lean_is_exclusive(x_20); -if (x_94 == 0) +uint8_t x_89; +lean_dec(x_18); +lean_dec(x_2); +x_89 = !lean_is_exclusive(x_19); +if (x_89 == 0) { -return x_20; +return x_19; } else { -lean_object* x_95; lean_object* x_96; lean_object* x_97; -x_95 = lean_ctor_get(x_20, 0); -x_96 = lean_ctor_get(x_20, 1); -lean_inc(x_96); -lean_inc(x_95); -lean_dec(x_20); -x_97 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_97, 0, x_95); -lean_ctor_set(x_97, 1, x_96); -return x_97; +lean_object* x_90; lean_object* x_91; lean_object* x_92; +x_90 = lean_ctor_get(x_19, 0); +x_91 = lean_ctor_get(x_19, 1); +lean_inc(x_91); +lean_inc(x_90); +lean_dec(x_19); +x_92 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_92, 0, x_90); +lean_ctor_set(x_92, 1, x_91); +return x_92; } } } } else { -uint8_t x_98; -lean_dec(x_8); +uint8_t x_93; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_98 = !lean_is_exclusive(x_10); -if (x_98 == 0) +lean_dec(x_2); +x_93 = !lean_is_exclusive(x_9); +if (x_93 == 0) { -return x_10; +return x_9; } else { -lean_object* x_99; lean_object* x_100; lean_object* x_101; -x_99 = lean_ctor_get(x_10, 0); -x_100 = lean_ctor_get(x_10, 1); -lean_inc(x_100); -lean_inc(x_99); -lean_dec(x_10); -x_101 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_101, 0, x_99); -lean_ctor_set(x_101, 1, x_100); -return x_101; +lean_object* x_94; lean_object* x_95; lean_object* x_96; +x_94 = lean_ctor_get(x_9, 0); +x_95 = lean_ctor_get(x_9, 1); +lean_inc(x_95); +lean_inc(x_94); +lean_dec(x_9); +x_96 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_96, 0, x_94); +lean_ctor_set(x_96, 1, x_95); +return x_96; } } } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__9___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__9___closed__1() { _start: { lean_object* x_1; @@ -3579,21 +3386,21 @@ x_1 = lean_mk_string_unchecked("append_congr", 12, 12); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__9___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__9___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__9___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__9___closed__1; x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { lean_object* x_17; lean_object* x_18; @@ -3642,7 +3449,7 @@ if (x_26 == 0) { lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; x_27 = lean_ctor_get(x_25, 0); -x_28 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__9___closed__2; +x_28 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__9___closed__2; x_29 = l_Lean_Expr_const___override(x_28, x_5); x_30 = l_Lean_mkApp8(x_29, x_6, x_7, x_8, x_10, x_9, x_27, x_19, x_23); lean_ctor_set(x_25, 0, x_30); @@ -3656,7 +3463,7 @@ x_32 = lean_ctor_get(x_25, 1); lean_inc(x_32); lean_inc(x_31); lean_dec(x_25); -x_33 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__9___closed__2; +x_33 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__9___closed__2; x_34 = l_Lean_Expr_const___override(x_33, x_5); x_35 = l_Lean_mkApp8(x_34, x_6, x_7, x_8, x_10, x_9, x_31, x_19, x_23); x_36 = lean_alloc_ctor(0, 2, 0); @@ -3740,7 +3547,7 @@ return x_44; } } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__1() { _start: { lean_object* x_1; @@ -3748,7 +3555,7 @@ x_1 = lean_mk_string_unchecked("append", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; @@ -3756,22 +3563,22 @@ x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__4; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__1; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__2; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__2; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; @@ -3781,7 +3588,7 @@ lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_1); -x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofOrAtom(x_1, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(x_1, x_3, x_4, x_5, x_6, x_7, x_8); if (lean_obj_tag(x_9) == 0) { lean_object* x_10; @@ -3830,7 +3637,7 @@ x_18 = lean_ctor_get(x_10, 0); lean_inc(x_18); lean_dec(x_10); lean_inc(x_2); -x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofOrAtom(x_2, x_3, x_4, x_5, x_6, x_7, x_17); +x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(x_2, x_3, x_4, x_5, x_6, x_7, x_17); if (lean_obj_tag(x_19) == 0) { lean_object* x_20; @@ -3903,7 +3710,7 @@ lean_inc(x_34); x_39 = l_Lean_mkNatLit(x_34); x_40 = lean_ctor_get(x_30, 3); lean_inc(x_40); -x_41 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__3; +x_41 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__3; lean_inc(x_40); lean_inc(x_33); lean_inc(x_39); @@ -3915,7 +3722,7 @@ lean_closure_set(x_43, 0, x_31); lean_closure_set(x_43, 1, x_33); lean_inc(x_34); lean_inc(x_18); -x_44 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__9), 16, 9); +x_44 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__9), 16, 9); lean_closure_set(x_44, 0, x_18); lean_closure_set(x_44, 1, x_30); lean_closure_set(x_44, 2, x_34); @@ -3999,7 +3806,7 @@ lean_inc(x_59); x_64 = l_Lean_mkNatLit(x_59); x_65 = lean_ctor_get(x_55, 3); lean_inc(x_65); -x_66 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__3; +x_66 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__3; lean_inc(x_65); lean_inc(x_58); lean_inc(x_64); @@ -4011,7 +3818,7 @@ lean_closure_set(x_68, 0, x_56); lean_closure_set(x_68, 1, x_58); lean_inc(x_59); lean_inc(x_18); -x_69 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__9), 16, 9); +x_69 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__9), 16, 9); lean_closure_set(x_69, 0, x_18); lean_closure_set(x_69, 1, x_55); lean_closure_set(x_69, 2, x_59); @@ -4091,7 +3898,7 @@ lean_inc(x_81); x_86 = l_Lean_mkNatLit(x_81); x_87 = lean_ctor_get(x_76, 3); lean_inc(x_87); -x_88 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__3; +x_88 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__3; lean_inc(x_87); lean_inc(x_80); lean_inc(x_86); @@ -4103,7 +3910,7 @@ lean_closure_set(x_90, 0, x_78); lean_closure_set(x_90, 1, x_80); lean_inc(x_81); lean_inc(x_18); -x_91 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__9), 16, 9); +x_91 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__9), 16, 9); lean_closure_set(x_91, 0, x_18); lean_closure_set(x_91, 1, x_76); lean_closure_set(x_91, 2, x_81); @@ -4209,7 +4016,7 @@ return x_105; } } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__11___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11___closed__1() { _start: { lean_object* x_1; @@ -4217,21 +4024,21 @@ x_1 = lean_mk_string_unchecked("signExtend_congr", 16, 16); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__11___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__11___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11___closed__1; x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__11(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; @@ -4247,7 +4054,7 @@ if (x_15 == 0) { lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; x_16 = lean_ctor_get(x_14, 0); -x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__11___closed__2; +x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11___closed__2; x_18 = l_Lean_Expr_const___override(x_17, x_2); x_19 = l_Lean_mkApp5(x_18, x_3, x_4, x_5, x_6, x_16); lean_ctor_set(x_14, 0, x_19); @@ -4261,7 +4068,7 @@ x_21 = lean_ctor_get(x_14, 1); lean_inc(x_21); lean_inc(x_20); lean_dec(x_14); -x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__11___closed__2; +x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11___closed__2; x_23 = l_Lean_Expr_const___override(x_22, x_2); x_24 = l_Lean_mkApp5(x_23, x_3, x_4, x_5, x_6, x_20); x_25 = lean_alloc_ctor(0, 2, 0); @@ -4299,7 +4106,7 @@ return x_29; } } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__1() { _start: { lean_object* x_1; @@ -4307,7 +4114,7 @@ x_1 = lean_mk_string_unchecked("signExtend", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; @@ -4315,394 +4122,371 @@ x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__4; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__1; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__2; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__2; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_10; -lean_inc(x_8); +lean_object* x_9; lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_10 = l_Lean_Meta_getNatValue_x3f(x_2, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_10) == 0) +lean_inc(x_4); +x_9 = l_Lean_Meta_getNatValue_x3f(x_1, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_9) == 0) { -lean_object* x_11; -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -if (lean_obj_tag(x_11) == 0) +lean_object* x_10; +x_10 = lean_ctor_get(x_9, 0); +lean_inc(x_10); +if (lean_obj_tag(x_10) == 0) { -lean_object* x_12; lean_object* x_13; +uint8_t x_11; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_12 = lean_ctor_get(x_10, 1); -lean_inc(x_12); -lean_dec(x_10); -x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_4, x_5, x_6, x_7, x_8, x_12); -if (lean_obj_tag(x_13) == 0) -{ -uint8_t x_14; -x_14 = !lean_is_exclusive(x_13); -if (x_14 == 0) -{ -return x_13; -} -else -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = lean_ctor_get(x_13, 0); -x_16 = lean_ctor_get(x_13, 1); -lean_inc(x_16); -lean_inc(x_15); -lean_dec(x_13); -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_15); -lean_ctor_set(x_17, 1, x_16); -return x_17; -} -} -else -{ -uint8_t x_18; -x_18 = !lean_is_exclusive(x_13); -if (x_18 == 0) +lean_dec(x_1); +x_11 = !lean_is_exclusive(x_9); +if (x_11 == 0) { -return x_13; +lean_object* x_12; lean_object* x_13; +x_12 = lean_ctor_get(x_9, 0); +lean_dec(x_12); +x_13 = lean_box(0); +lean_ctor_set(x_9, 0, x_13); +return x_9; } else { -lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_19 = lean_ctor_get(x_13, 0); -x_20 = lean_ctor_get(x_13, 1); -lean_inc(x_20); -lean_inc(x_19); -lean_dec(x_13); -x_21 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_21, 0, x_19); -lean_ctor_set(x_21, 1, x_20); -return x_21; -} +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_9, 1); +lean_inc(x_14); +lean_dec(x_9); +x_15 = lean_box(0); +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_16, 1, x_14); +return x_16; } } else { -lean_object* x_22; lean_object* x_23; lean_object* x_24; -lean_dec(x_1); -x_22 = lean_ctor_get(x_10, 1); -lean_inc(x_22); +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_9, 1); +lean_inc(x_17); +lean_dec(x_9); +x_18 = lean_ctor_get(x_10, 0); +lean_inc(x_18); lean_dec(x_10); -x_23 = lean_ctor_get(x_11, 0); -lean_inc(x_23); -lean_dec(x_11); -lean_inc(x_3); -x_24 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofOrAtom(x_3, x_4, x_5, x_6, x_7, x_8, x_22); -if (lean_obj_tag(x_24) == 0) +lean_inc(x_2); +x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(x_2, x_3, x_4, x_5, x_6, x_7, x_17); +if (lean_obj_tag(x_19) == 0) { -lean_object* x_25; -x_25 = lean_ctor_get(x_24, 0); -lean_inc(x_25); -if (lean_obj_tag(x_25) == 0) +lean_object* x_20; +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +if (lean_obj_tag(x_20) == 0) { -uint8_t x_26; -lean_dec(x_23); -lean_dec(x_3); +uint8_t x_21; +lean_dec(x_18); lean_dec(x_2); -x_26 = !lean_is_exclusive(x_24); -if (x_26 == 0) +lean_dec(x_1); +x_21 = !lean_is_exclusive(x_19); +if (x_21 == 0) { -lean_object* x_27; lean_object* x_28; -x_27 = lean_ctor_get(x_24, 0); -lean_dec(x_27); -x_28 = lean_box(0); -lean_ctor_set(x_24, 0, x_28); -return x_24; +lean_object* x_22; lean_object* x_23; +x_22 = lean_ctor_get(x_19, 0); +lean_dec(x_22); +x_23 = lean_box(0); +lean_ctor_set(x_19, 0, x_23); +return x_19; } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_24, 1); -lean_inc(x_29); -lean_dec(x_24); -x_30 = lean_box(0); -x_31 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_31, 0, x_30); -lean_ctor_set(x_31, 1, x_29); -return x_31; +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_19, 1); +lean_inc(x_24); +lean_dec(x_19); +x_25 = lean_box(0); +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_24); +return x_26; } } else { -uint8_t x_32; -x_32 = !lean_is_exclusive(x_25); -if (x_32 == 0) +uint8_t x_27; +x_27 = !lean_is_exclusive(x_20); +if (x_27 == 0) { -uint8_t x_33; -x_33 = !lean_is_exclusive(x_24); -if (x_33 == 0) +uint8_t x_28; +x_28 = !lean_is_exclusive(x_19); +if (x_28 == 0) { -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; uint8_t x_46; -x_34 = lean_ctor_get(x_25, 0); -x_35 = lean_ctor_get(x_24, 0); -lean_dec(x_35); -x_36 = lean_ctor_get(x_34, 0); -lean_inc(x_36); -x_37 = lean_ctor_get(x_34, 1); -lean_inc(x_37); -x_38 = lean_ctor_get(x_34, 3); -lean_inc(x_38); -lean_inc(x_23); -lean_inc(x_36); -x_39 = lean_alloc_ctor(8, 3, 0); -lean_ctor_set(x_39, 0, x_36); -lean_ctor_set(x_39, 1, x_23); -lean_ctor_set(x_39, 2, x_37); -x_40 = lean_box(0); +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; +x_29 = lean_ctor_get(x_20, 0); +x_30 = lean_ctor_get(x_19, 0); +lean_dec(x_30); +x_31 = lean_ctor_get(x_29, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_29, 1); +lean_inc(x_32); +x_33 = lean_ctor_get(x_29, 3); +lean_inc(x_33); +lean_inc(x_18); +lean_inc(x_31); +x_34 = lean_alloc_ctor(8, 3, 0); +lean_ctor_set(x_34, 0, x_31); +lean_ctor_set(x_34, 1, x_18); +lean_ctor_set(x_34, 2, x_32); +x_35 = lean_box(0); +lean_inc(x_31); +x_36 = l_Lean_mkNatLit(x_31); +x_37 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__3; +lean_inc(x_33); +lean_inc(x_1); lean_inc(x_36); -x_41 = l_Lean_mkNatLit(x_36); -x_42 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__3; -lean_inc(x_38); -lean_inc(x_2); -lean_inc(x_41); -x_43 = l_Lean_mkApp3(x_42, x_41, x_2, x_38); -x_44 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_44, 0, x_36); -lean_closure_set(x_44, 1, x_38); -lean_inc(x_34); -x_45 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__11), 12, 5); -lean_closure_set(x_45, 0, x_34); -lean_closure_set(x_45, 1, x_40); -lean_closure_set(x_45, 2, x_2); -lean_closure_set(x_45, 3, x_41); -lean_closure_set(x_45, 4, x_3); -x_46 = !lean_is_exclusive(x_34); -if (x_46 == 0) -{ -lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_47 = lean_ctor_get(x_34, 3); -lean_dec(x_47); -x_48 = lean_ctor_get(x_34, 2); -lean_dec(x_48); -x_49 = lean_ctor_get(x_34, 1); -lean_dec(x_49); -x_50 = lean_ctor_get(x_34, 0); -lean_dec(x_50); -x_51 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_51, 0, x_44); -lean_closure_set(x_51, 1, x_45); -lean_ctor_set(x_34, 3, x_43); -lean_ctor_set(x_34, 2, x_51); -lean_ctor_set(x_34, 1, x_39); -lean_ctor_set(x_34, 0, x_23); -return x_24; +x_38 = l_Lean_mkApp3(x_37, x_36, x_1, x_33); +x_39 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_39, 0, x_31); +lean_closure_set(x_39, 1, x_33); +lean_inc(x_29); +x_40 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11), 12, 5); +lean_closure_set(x_40, 0, x_29); +lean_closure_set(x_40, 1, x_35); +lean_closure_set(x_40, 2, x_1); +lean_closure_set(x_40, 3, x_36); +lean_closure_set(x_40, 4, x_2); +x_41 = !lean_is_exclusive(x_29); +if (x_41 == 0) +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_42 = lean_ctor_get(x_29, 3); +lean_dec(x_42); +x_43 = lean_ctor_get(x_29, 2); +lean_dec(x_43); +x_44 = lean_ctor_get(x_29, 1); +lean_dec(x_44); +x_45 = lean_ctor_get(x_29, 0); +lean_dec(x_45); +x_46 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_46, 0, x_39); +lean_closure_set(x_46, 1, x_40); +lean_ctor_set(x_29, 3, x_38); +lean_ctor_set(x_29, 2, x_46); +lean_ctor_set(x_29, 1, x_34); +lean_ctor_set(x_29, 0, x_18); +return x_19; } else { -lean_object* x_52; lean_object* x_53; -lean_dec(x_34); -x_52 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_52, 0, x_44); -lean_closure_set(x_52, 1, x_45); -x_53 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_53, 0, x_23); -lean_ctor_set(x_53, 1, x_39); -lean_ctor_set(x_53, 2, x_52); -lean_ctor_set(x_53, 3, x_43); -lean_ctor_set(x_25, 0, x_53); -return x_24; +lean_object* x_47; lean_object* x_48; +lean_dec(x_29); +x_47 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_47, 0, x_39); +lean_closure_set(x_47, 1, x_40); +x_48 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_48, 0, x_18); +lean_ctor_set(x_48, 1, x_34); +lean_ctor_set(x_48, 2, x_47); +lean_ctor_set(x_48, 3, x_38); +lean_ctor_set(x_20, 0, x_48); +return x_19; } } else { -lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_54 = lean_ctor_get(x_25, 0); -x_55 = lean_ctor_get(x_24, 1); -lean_inc(x_55); -lean_dec(x_24); -x_56 = lean_ctor_get(x_54, 0); -lean_inc(x_56); -x_57 = lean_ctor_get(x_54, 1); -lean_inc(x_57); -x_58 = lean_ctor_get(x_54, 3); -lean_inc(x_58); -lean_inc(x_23); -lean_inc(x_56); -x_59 = lean_alloc_ctor(8, 3, 0); -lean_ctor_set(x_59, 0, x_56); -lean_ctor_set(x_59, 1, x_23); -lean_ctor_set(x_59, 2, x_57); -x_60 = lean_box(0); +lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; +x_49 = lean_ctor_get(x_20, 0); +x_50 = lean_ctor_get(x_19, 1); +lean_inc(x_50); +lean_dec(x_19); +x_51 = lean_ctor_get(x_49, 0); +lean_inc(x_51); +x_52 = lean_ctor_get(x_49, 1); +lean_inc(x_52); +x_53 = lean_ctor_get(x_49, 3); +lean_inc(x_53); +lean_inc(x_18); +lean_inc(x_51); +x_54 = lean_alloc_ctor(8, 3, 0); +lean_ctor_set(x_54, 0, x_51); +lean_ctor_set(x_54, 1, x_18); +lean_ctor_set(x_54, 2, x_52); +x_55 = lean_box(0); +lean_inc(x_51); +x_56 = l_Lean_mkNatLit(x_51); +x_57 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__3; +lean_inc(x_53); +lean_inc(x_1); lean_inc(x_56); -x_61 = l_Lean_mkNatLit(x_56); -x_62 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__3; -lean_inc(x_58); -lean_inc(x_2); -lean_inc(x_61); -x_63 = l_Lean_mkApp3(x_62, x_61, x_2, x_58); -x_64 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_64, 0, x_56); -lean_closure_set(x_64, 1, x_58); -lean_inc(x_54); -x_65 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__11), 12, 5); -lean_closure_set(x_65, 0, x_54); -lean_closure_set(x_65, 1, x_60); -lean_closure_set(x_65, 2, x_2); -lean_closure_set(x_65, 3, x_61); -lean_closure_set(x_65, 4, x_3); -if (lean_is_exclusive(x_54)) { - lean_ctor_release(x_54, 0); - lean_ctor_release(x_54, 1); - lean_ctor_release(x_54, 2); - lean_ctor_release(x_54, 3); - x_66 = x_54; +x_58 = l_Lean_mkApp3(x_57, x_56, x_1, x_53); +x_59 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_59, 0, x_51); +lean_closure_set(x_59, 1, x_53); +lean_inc(x_49); +x_60 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11), 12, 5); +lean_closure_set(x_60, 0, x_49); +lean_closure_set(x_60, 1, x_55); +lean_closure_set(x_60, 2, x_1); +lean_closure_set(x_60, 3, x_56); +lean_closure_set(x_60, 4, x_2); +if (lean_is_exclusive(x_49)) { + lean_ctor_release(x_49, 0); + lean_ctor_release(x_49, 1); + lean_ctor_release(x_49, 2); + lean_ctor_release(x_49, 3); + x_61 = x_49; } else { - lean_dec_ref(x_54); - x_66 = lean_box(0); -} -x_67 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_67, 0, x_64); -lean_closure_set(x_67, 1, x_65); -if (lean_is_scalar(x_66)) { - x_68 = lean_alloc_ctor(0, 4, 0); + lean_dec_ref(x_49); + x_61 = lean_box(0); +} +x_62 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_62, 0, x_59); +lean_closure_set(x_62, 1, x_60); +if (lean_is_scalar(x_61)) { + x_63 = lean_alloc_ctor(0, 4, 0); } else { - x_68 = x_66; + x_63 = x_61; } -lean_ctor_set(x_68, 0, x_23); -lean_ctor_set(x_68, 1, x_59); -lean_ctor_set(x_68, 2, x_67); -lean_ctor_set(x_68, 3, x_63); -lean_ctor_set(x_25, 0, x_68); -x_69 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_69, 0, x_25); -lean_ctor_set(x_69, 1, x_55); -return x_69; +lean_ctor_set(x_63, 0, x_18); +lean_ctor_set(x_63, 1, x_54); +lean_ctor_set(x_63, 2, x_62); +lean_ctor_set(x_63, 3, x_58); +lean_ctor_set(x_20, 0, x_63); +x_64 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_64, 0, x_20); +lean_ctor_set(x_64, 1, x_50); +return x_64; } } else { -lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; -x_70 = lean_ctor_get(x_25, 0); -lean_inc(x_70); -lean_dec(x_25); -x_71 = lean_ctor_get(x_24, 1); -lean_inc(x_71); -if (lean_is_exclusive(x_24)) { - lean_ctor_release(x_24, 0); - lean_ctor_release(x_24, 1); - x_72 = x_24; +lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; +x_65 = lean_ctor_get(x_20, 0); +lean_inc(x_65); +lean_dec(x_20); +x_66 = lean_ctor_get(x_19, 1); +lean_inc(x_66); +if (lean_is_exclusive(x_19)) { + lean_ctor_release(x_19, 0); + lean_ctor_release(x_19, 1); + x_67 = x_19; } else { - lean_dec_ref(x_24); - x_72 = lean_box(0); + lean_dec_ref(x_19); + x_67 = lean_box(0); } -x_73 = lean_ctor_get(x_70, 0); -lean_inc(x_73); -x_74 = lean_ctor_get(x_70, 1); -lean_inc(x_74); -x_75 = lean_ctor_get(x_70, 3); -lean_inc(x_75); -lean_inc(x_23); -lean_inc(x_73); -x_76 = lean_alloc_ctor(8, 3, 0); -lean_ctor_set(x_76, 0, x_73); -lean_ctor_set(x_76, 1, x_23); -lean_ctor_set(x_76, 2, x_74); -x_77 = lean_box(0); -lean_inc(x_73); -x_78 = l_Lean_mkNatLit(x_73); -x_79 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__3; -lean_inc(x_75); -lean_inc(x_2); -lean_inc(x_78); -x_80 = l_Lean_mkApp3(x_79, x_78, x_2, x_75); -x_81 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_81, 0, x_73); -lean_closure_set(x_81, 1, x_75); +x_68 = lean_ctor_get(x_65, 0); +lean_inc(x_68); +x_69 = lean_ctor_get(x_65, 1); +lean_inc(x_69); +x_70 = lean_ctor_get(x_65, 3); lean_inc(x_70); -x_82 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__11), 12, 5); -lean_closure_set(x_82, 0, x_70); -lean_closure_set(x_82, 1, x_77); -lean_closure_set(x_82, 2, x_2); -lean_closure_set(x_82, 3, x_78); -lean_closure_set(x_82, 4, x_3); -if (lean_is_exclusive(x_70)) { - lean_ctor_release(x_70, 0); - lean_ctor_release(x_70, 1); - lean_ctor_release(x_70, 2); - lean_ctor_release(x_70, 3); - x_83 = x_70; +lean_inc(x_18); +lean_inc(x_68); +x_71 = lean_alloc_ctor(8, 3, 0); +lean_ctor_set(x_71, 0, x_68); +lean_ctor_set(x_71, 1, x_18); +lean_ctor_set(x_71, 2, x_69); +x_72 = lean_box(0); +lean_inc(x_68); +x_73 = l_Lean_mkNatLit(x_68); +x_74 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__3; +lean_inc(x_70); +lean_inc(x_1); +lean_inc(x_73); +x_75 = l_Lean_mkApp3(x_74, x_73, x_1, x_70); +x_76 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_76, 0, x_68); +lean_closure_set(x_76, 1, x_70); +lean_inc(x_65); +x_77 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11), 12, 5); +lean_closure_set(x_77, 0, x_65); +lean_closure_set(x_77, 1, x_72); +lean_closure_set(x_77, 2, x_1); +lean_closure_set(x_77, 3, x_73); +lean_closure_set(x_77, 4, x_2); +if (lean_is_exclusive(x_65)) { + lean_ctor_release(x_65, 0); + lean_ctor_release(x_65, 1); + lean_ctor_release(x_65, 2); + lean_ctor_release(x_65, 3); + x_78 = x_65; } else { - lean_dec_ref(x_70); - x_83 = lean_box(0); + lean_dec_ref(x_65); + x_78 = lean_box(0); } -x_84 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_84, 0, x_81); -lean_closure_set(x_84, 1, x_82); -if (lean_is_scalar(x_83)) { - x_85 = lean_alloc_ctor(0, 4, 0); +x_79 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_79, 0, x_76); +lean_closure_set(x_79, 1, x_77); +if (lean_is_scalar(x_78)) { + x_80 = lean_alloc_ctor(0, 4, 0); } else { - x_85 = x_83; -} -lean_ctor_set(x_85, 0, x_23); -lean_ctor_set(x_85, 1, x_76); -lean_ctor_set(x_85, 2, x_84); -lean_ctor_set(x_85, 3, x_80); -x_86 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_86, 0, x_85); -if (lean_is_scalar(x_72)) { - x_87 = lean_alloc_ctor(0, 2, 0); + x_80 = x_78; +} +lean_ctor_set(x_80, 0, x_18); +lean_ctor_set(x_80, 1, x_71); +lean_ctor_set(x_80, 2, x_79); +lean_ctor_set(x_80, 3, x_75); +x_81 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_81, 0, x_80); +if (lean_is_scalar(x_67)) { + x_82 = lean_alloc_ctor(0, 2, 0); } else { - x_87 = x_72; + x_82 = x_67; } -lean_ctor_set(x_87, 0, x_86); -lean_ctor_set(x_87, 1, x_71); -return x_87; +lean_ctor_set(x_82, 0, x_81); +lean_ctor_set(x_82, 1, x_66); +return x_82; } } } else { -uint8_t x_88; -lean_dec(x_23); -lean_dec(x_3); +uint8_t x_83; +lean_dec(x_18); lean_dec(x_2); -x_88 = !lean_is_exclusive(x_24); -if (x_88 == 0) +lean_dec(x_1); +x_83 = !lean_is_exclusive(x_19); +if (x_83 == 0) { -return x_24; +return x_19; } else { -lean_object* x_89; lean_object* x_90; lean_object* x_91; -x_89 = lean_ctor_get(x_24, 0); -x_90 = lean_ctor_get(x_24, 1); -lean_inc(x_90); -lean_inc(x_89); -lean_dec(x_24); -x_91 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_91, 0, x_89); -lean_ctor_set(x_91, 1, x_90); -return x_91; +lean_object* x_84; lean_object* x_85; lean_object* x_86; +x_84 = lean_ctor_get(x_19, 0); +x_85 = lean_ctor_get(x_19, 1); +lean_inc(x_85); +lean_inc(x_84); +lean_dec(x_19); +x_86 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_86, 0, x_84); +lean_ctor_set(x_86, 1, x_85); +return x_86; } } } } else { -uint8_t x_92; -lean_dec(x_8); +uint8_t x_87; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -4710,28 +4494,28 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_92 = !lean_is_exclusive(x_10); -if (x_92 == 0) +x_87 = !lean_is_exclusive(x_9); +if (x_87 == 0) { -return x_10; +return x_9; } else { -lean_object* x_93; lean_object* x_94; lean_object* x_95; -x_93 = lean_ctor_get(x_10, 0); -x_94 = lean_ctor_get(x_10, 1); -lean_inc(x_94); -lean_inc(x_93); -lean_dec(x_10); -x_95 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_95, 0, x_93); -lean_ctor_set(x_95, 1, x_94); -return x_95; +lean_object* x_88; lean_object* x_89; lean_object* x_90; +x_88 = lean_ctor_get(x_9, 0); +x_89 = lean_ctor_get(x_9, 1); +lean_inc(x_89); +lean_inc(x_88); +lean_dec(x_9); +x_90 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_90, 0, x_88); +lean_ctor_set(x_90, 1, x_89); +return x_90; } } } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13___closed__1() { _start: { lean_object* x_1; @@ -4739,21 +4523,21 @@ x_1 = lean_mk_string_unchecked("zeroExtend_congr", 16, 16); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13___closed__1; x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; @@ -4769,7 +4553,7 @@ if (x_15 == 0) { lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; x_16 = lean_ctor_get(x_14, 0); -x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13___closed__2; +x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13___closed__2; x_18 = l_Lean_Expr_const___override(x_17, x_2); x_19 = l_Lean_mkApp5(x_18, x_3, x_4, x_5, x_6, x_16); lean_ctor_set(x_14, 0, x_19); @@ -4783,7 +4567,7 @@ x_21 = lean_ctor_get(x_14, 1); lean_inc(x_21); lean_inc(x_20); lean_dec(x_14); -x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13___closed__2; +x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13___closed__2; x_23 = l_Lean_Expr_const___override(x_22, x_2); x_24 = l_Lean_mkApp5(x_23, x_3, x_4, x_5, x_6, x_20); x_25 = lean_alloc_ctor(0, 2, 0); @@ -4821,7 +4605,7 @@ return x_29; } } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__1() { _start: { lean_object* x_1; @@ -4829,7 +4613,7 @@ x_1 = lean_mk_string_unchecked("zeroExtend", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; @@ -4837,394 +4621,371 @@ x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__4; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__1; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__2; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__2; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_10; -lean_inc(x_8); +lean_object* x_9; lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_10 = l_Lean_Meta_getNatValue_x3f(x_2, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_10) == 0) +lean_inc(x_4); +x_9 = l_Lean_Meta_getNatValue_x3f(x_1, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_9) == 0) { -lean_object* x_11; -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -if (lean_obj_tag(x_11) == 0) +lean_object* x_10; +x_10 = lean_ctor_get(x_9, 0); +lean_inc(x_10); +if (lean_obj_tag(x_10) == 0) { -lean_object* x_12; lean_object* x_13; +uint8_t x_11; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_12 = lean_ctor_get(x_10, 1); -lean_inc(x_12); -lean_dec(x_10); -x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_4, x_5, x_6, x_7, x_8, x_12); -if (lean_obj_tag(x_13) == 0) -{ -uint8_t x_14; -x_14 = !lean_is_exclusive(x_13); -if (x_14 == 0) -{ -return x_13; -} -else -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = lean_ctor_get(x_13, 0); -x_16 = lean_ctor_get(x_13, 1); -lean_inc(x_16); -lean_inc(x_15); -lean_dec(x_13); -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_15); -lean_ctor_set(x_17, 1, x_16); -return x_17; -} -} -else -{ -uint8_t x_18; -x_18 = !lean_is_exclusive(x_13); -if (x_18 == 0) +lean_dec(x_1); +x_11 = !lean_is_exclusive(x_9); +if (x_11 == 0) { -return x_13; +lean_object* x_12; lean_object* x_13; +x_12 = lean_ctor_get(x_9, 0); +lean_dec(x_12); +x_13 = lean_box(0); +lean_ctor_set(x_9, 0, x_13); +return x_9; } else { -lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_19 = lean_ctor_get(x_13, 0); -x_20 = lean_ctor_get(x_13, 1); -lean_inc(x_20); -lean_inc(x_19); -lean_dec(x_13); -x_21 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_21, 0, x_19); -lean_ctor_set(x_21, 1, x_20); -return x_21; -} +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_9, 1); +lean_inc(x_14); +lean_dec(x_9); +x_15 = lean_box(0); +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_16, 1, x_14); +return x_16; } } else { -lean_object* x_22; lean_object* x_23; lean_object* x_24; -lean_dec(x_1); -x_22 = lean_ctor_get(x_10, 1); -lean_inc(x_22); +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_9, 1); +lean_inc(x_17); +lean_dec(x_9); +x_18 = lean_ctor_get(x_10, 0); +lean_inc(x_18); lean_dec(x_10); -x_23 = lean_ctor_get(x_11, 0); -lean_inc(x_23); -lean_dec(x_11); -lean_inc(x_3); -x_24 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofOrAtom(x_3, x_4, x_5, x_6, x_7, x_8, x_22); -if (lean_obj_tag(x_24) == 0) +lean_inc(x_2); +x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(x_2, x_3, x_4, x_5, x_6, x_7, x_17); +if (lean_obj_tag(x_19) == 0) { -lean_object* x_25; -x_25 = lean_ctor_get(x_24, 0); -lean_inc(x_25); -if (lean_obj_tag(x_25) == 0) +lean_object* x_20; +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +if (lean_obj_tag(x_20) == 0) { -uint8_t x_26; -lean_dec(x_23); -lean_dec(x_3); +uint8_t x_21; +lean_dec(x_18); lean_dec(x_2); -x_26 = !lean_is_exclusive(x_24); -if (x_26 == 0) +lean_dec(x_1); +x_21 = !lean_is_exclusive(x_19); +if (x_21 == 0) { -lean_object* x_27; lean_object* x_28; -x_27 = lean_ctor_get(x_24, 0); -lean_dec(x_27); -x_28 = lean_box(0); -lean_ctor_set(x_24, 0, x_28); -return x_24; +lean_object* x_22; lean_object* x_23; +x_22 = lean_ctor_get(x_19, 0); +lean_dec(x_22); +x_23 = lean_box(0); +lean_ctor_set(x_19, 0, x_23); +return x_19; } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_24, 1); -lean_inc(x_29); -lean_dec(x_24); -x_30 = lean_box(0); -x_31 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_31, 0, x_30); -lean_ctor_set(x_31, 1, x_29); -return x_31; +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_19, 1); +lean_inc(x_24); +lean_dec(x_19); +x_25 = lean_box(0); +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_24); +return x_26; } } else { -uint8_t x_32; -x_32 = !lean_is_exclusive(x_25); -if (x_32 == 0) +uint8_t x_27; +x_27 = !lean_is_exclusive(x_20); +if (x_27 == 0) { -uint8_t x_33; -x_33 = !lean_is_exclusive(x_24); -if (x_33 == 0) +uint8_t x_28; +x_28 = !lean_is_exclusive(x_19); +if (x_28 == 0) { -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; uint8_t x_46; -x_34 = lean_ctor_get(x_25, 0); -x_35 = lean_ctor_get(x_24, 0); -lean_dec(x_35); -x_36 = lean_ctor_get(x_34, 0); -lean_inc(x_36); -x_37 = lean_ctor_get(x_34, 1); -lean_inc(x_37); -x_38 = lean_ctor_get(x_34, 3); -lean_inc(x_38); -lean_inc(x_23); -lean_inc(x_36); -x_39 = lean_alloc_ctor(2, 3, 0); -lean_ctor_set(x_39, 0, x_36); -lean_ctor_set(x_39, 1, x_23); -lean_ctor_set(x_39, 2, x_37); -x_40 = lean_box(0); +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; +x_29 = lean_ctor_get(x_20, 0); +x_30 = lean_ctor_get(x_19, 0); +lean_dec(x_30); +x_31 = lean_ctor_get(x_29, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_29, 1); +lean_inc(x_32); +x_33 = lean_ctor_get(x_29, 3); +lean_inc(x_33); +lean_inc(x_18); +lean_inc(x_31); +x_34 = lean_alloc_ctor(2, 3, 0); +lean_ctor_set(x_34, 0, x_31); +lean_ctor_set(x_34, 1, x_18); +lean_ctor_set(x_34, 2, x_32); +x_35 = lean_box(0); +lean_inc(x_31); +x_36 = l_Lean_mkNatLit(x_31); +x_37 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__3; +lean_inc(x_33); +lean_inc(x_1); lean_inc(x_36); -x_41 = l_Lean_mkNatLit(x_36); -x_42 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__3; -lean_inc(x_38); -lean_inc(x_2); -lean_inc(x_41); -x_43 = l_Lean_mkApp3(x_42, x_41, x_2, x_38); -x_44 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_44, 0, x_36); -lean_closure_set(x_44, 1, x_38); -lean_inc(x_34); -x_45 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13), 12, 5); -lean_closure_set(x_45, 0, x_34); -lean_closure_set(x_45, 1, x_40); -lean_closure_set(x_45, 2, x_2); -lean_closure_set(x_45, 3, x_41); -lean_closure_set(x_45, 4, x_3); -x_46 = !lean_is_exclusive(x_34); -if (x_46 == 0) -{ -lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_47 = lean_ctor_get(x_34, 3); -lean_dec(x_47); -x_48 = lean_ctor_get(x_34, 2); -lean_dec(x_48); -x_49 = lean_ctor_get(x_34, 1); -lean_dec(x_49); -x_50 = lean_ctor_get(x_34, 0); -lean_dec(x_50); -x_51 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_51, 0, x_44); -lean_closure_set(x_51, 1, x_45); -lean_ctor_set(x_34, 3, x_43); -lean_ctor_set(x_34, 2, x_51); -lean_ctor_set(x_34, 1, x_39); -lean_ctor_set(x_34, 0, x_23); -return x_24; +x_38 = l_Lean_mkApp3(x_37, x_36, x_1, x_33); +x_39 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_39, 0, x_31); +lean_closure_set(x_39, 1, x_33); +lean_inc(x_29); +x_40 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13), 12, 5); +lean_closure_set(x_40, 0, x_29); +lean_closure_set(x_40, 1, x_35); +lean_closure_set(x_40, 2, x_1); +lean_closure_set(x_40, 3, x_36); +lean_closure_set(x_40, 4, x_2); +x_41 = !lean_is_exclusive(x_29); +if (x_41 == 0) +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_42 = lean_ctor_get(x_29, 3); +lean_dec(x_42); +x_43 = lean_ctor_get(x_29, 2); +lean_dec(x_43); +x_44 = lean_ctor_get(x_29, 1); +lean_dec(x_44); +x_45 = lean_ctor_get(x_29, 0); +lean_dec(x_45); +x_46 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_46, 0, x_39); +lean_closure_set(x_46, 1, x_40); +lean_ctor_set(x_29, 3, x_38); +lean_ctor_set(x_29, 2, x_46); +lean_ctor_set(x_29, 1, x_34); +lean_ctor_set(x_29, 0, x_18); +return x_19; } else { -lean_object* x_52; lean_object* x_53; -lean_dec(x_34); -x_52 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_52, 0, x_44); -lean_closure_set(x_52, 1, x_45); -x_53 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_53, 0, x_23); -lean_ctor_set(x_53, 1, x_39); -lean_ctor_set(x_53, 2, x_52); -lean_ctor_set(x_53, 3, x_43); -lean_ctor_set(x_25, 0, x_53); -return x_24; +lean_object* x_47; lean_object* x_48; +lean_dec(x_29); +x_47 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_47, 0, x_39); +lean_closure_set(x_47, 1, x_40); +x_48 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_48, 0, x_18); +lean_ctor_set(x_48, 1, x_34); +lean_ctor_set(x_48, 2, x_47); +lean_ctor_set(x_48, 3, x_38); +lean_ctor_set(x_20, 0, x_48); +return x_19; } } else { -lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_54 = lean_ctor_get(x_25, 0); -x_55 = lean_ctor_get(x_24, 1); -lean_inc(x_55); -lean_dec(x_24); -x_56 = lean_ctor_get(x_54, 0); -lean_inc(x_56); -x_57 = lean_ctor_get(x_54, 1); -lean_inc(x_57); -x_58 = lean_ctor_get(x_54, 3); -lean_inc(x_58); -lean_inc(x_23); -lean_inc(x_56); -x_59 = lean_alloc_ctor(2, 3, 0); -lean_ctor_set(x_59, 0, x_56); -lean_ctor_set(x_59, 1, x_23); -lean_ctor_set(x_59, 2, x_57); -x_60 = lean_box(0); +lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; +x_49 = lean_ctor_get(x_20, 0); +x_50 = lean_ctor_get(x_19, 1); +lean_inc(x_50); +lean_dec(x_19); +x_51 = lean_ctor_get(x_49, 0); +lean_inc(x_51); +x_52 = lean_ctor_get(x_49, 1); +lean_inc(x_52); +x_53 = lean_ctor_get(x_49, 3); +lean_inc(x_53); +lean_inc(x_18); +lean_inc(x_51); +x_54 = lean_alloc_ctor(2, 3, 0); +lean_ctor_set(x_54, 0, x_51); +lean_ctor_set(x_54, 1, x_18); +lean_ctor_set(x_54, 2, x_52); +x_55 = lean_box(0); +lean_inc(x_51); +x_56 = l_Lean_mkNatLit(x_51); +x_57 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__3; +lean_inc(x_53); +lean_inc(x_1); lean_inc(x_56); -x_61 = l_Lean_mkNatLit(x_56); -x_62 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__3; -lean_inc(x_58); -lean_inc(x_2); -lean_inc(x_61); -x_63 = l_Lean_mkApp3(x_62, x_61, x_2, x_58); -x_64 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_64, 0, x_56); -lean_closure_set(x_64, 1, x_58); -lean_inc(x_54); -x_65 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13), 12, 5); -lean_closure_set(x_65, 0, x_54); -lean_closure_set(x_65, 1, x_60); -lean_closure_set(x_65, 2, x_2); -lean_closure_set(x_65, 3, x_61); -lean_closure_set(x_65, 4, x_3); -if (lean_is_exclusive(x_54)) { - lean_ctor_release(x_54, 0); - lean_ctor_release(x_54, 1); - lean_ctor_release(x_54, 2); - lean_ctor_release(x_54, 3); - x_66 = x_54; +x_58 = l_Lean_mkApp3(x_57, x_56, x_1, x_53); +x_59 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_59, 0, x_51); +lean_closure_set(x_59, 1, x_53); +lean_inc(x_49); +x_60 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13), 12, 5); +lean_closure_set(x_60, 0, x_49); +lean_closure_set(x_60, 1, x_55); +lean_closure_set(x_60, 2, x_1); +lean_closure_set(x_60, 3, x_56); +lean_closure_set(x_60, 4, x_2); +if (lean_is_exclusive(x_49)) { + lean_ctor_release(x_49, 0); + lean_ctor_release(x_49, 1); + lean_ctor_release(x_49, 2); + lean_ctor_release(x_49, 3); + x_61 = x_49; } else { - lean_dec_ref(x_54); - x_66 = lean_box(0); -} -x_67 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_67, 0, x_64); -lean_closure_set(x_67, 1, x_65); -if (lean_is_scalar(x_66)) { - x_68 = lean_alloc_ctor(0, 4, 0); + lean_dec_ref(x_49); + x_61 = lean_box(0); +} +x_62 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_62, 0, x_59); +lean_closure_set(x_62, 1, x_60); +if (lean_is_scalar(x_61)) { + x_63 = lean_alloc_ctor(0, 4, 0); } else { - x_68 = x_66; + x_63 = x_61; } -lean_ctor_set(x_68, 0, x_23); -lean_ctor_set(x_68, 1, x_59); -lean_ctor_set(x_68, 2, x_67); -lean_ctor_set(x_68, 3, x_63); -lean_ctor_set(x_25, 0, x_68); -x_69 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_69, 0, x_25); -lean_ctor_set(x_69, 1, x_55); -return x_69; +lean_ctor_set(x_63, 0, x_18); +lean_ctor_set(x_63, 1, x_54); +lean_ctor_set(x_63, 2, x_62); +lean_ctor_set(x_63, 3, x_58); +lean_ctor_set(x_20, 0, x_63); +x_64 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_64, 0, x_20); +lean_ctor_set(x_64, 1, x_50); +return x_64; } } else { -lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; -x_70 = lean_ctor_get(x_25, 0); -lean_inc(x_70); -lean_dec(x_25); -x_71 = lean_ctor_get(x_24, 1); -lean_inc(x_71); -if (lean_is_exclusive(x_24)) { - lean_ctor_release(x_24, 0); - lean_ctor_release(x_24, 1); - x_72 = x_24; +lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; +x_65 = lean_ctor_get(x_20, 0); +lean_inc(x_65); +lean_dec(x_20); +x_66 = lean_ctor_get(x_19, 1); +lean_inc(x_66); +if (lean_is_exclusive(x_19)) { + lean_ctor_release(x_19, 0); + lean_ctor_release(x_19, 1); + x_67 = x_19; } else { - lean_dec_ref(x_24); - x_72 = lean_box(0); + lean_dec_ref(x_19); + x_67 = lean_box(0); } -x_73 = lean_ctor_get(x_70, 0); -lean_inc(x_73); -x_74 = lean_ctor_get(x_70, 1); -lean_inc(x_74); -x_75 = lean_ctor_get(x_70, 3); -lean_inc(x_75); -lean_inc(x_23); -lean_inc(x_73); -x_76 = lean_alloc_ctor(2, 3, 0); -lean_ctor_set(x_76, 0, x_73); -lean_ctor_set(x_76, 1, x_23); -lean_ctor_set(x_76, 2, x_74); -x_77 = lean_box(0); -lean_inc(x_73); -x_78 = l_Lean_mkNatLit(x_73); -x_79 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__3; -lean_inc(x_75); -lean_inc(x_2); -lean_inc(x_78); -x_80 = l_Lean_mkApp3(x_79, x_78, x_2, x_75); -x_81 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_81, 0, x_73); -lean_closure_set(x_81, 1, x_75); +x_68 = lean_ctor_get(x_65, 0); +lean_inc(x_68); +x_69 = lean_ctor_get(x_65, 1); +lean_inc(x_69); +x_70 = lean_ctor_get(x_65, 3); lean_inc(x_70); -x_82 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13), 12, 5); -lean_closure_set(x_82, 0, x_70); -lean_closure_set(x_82, 1, x_77); -lean_closure_set(x_82, 2, x_2); -lean_closure_set(x_82, 3, x_78); -lean_closure_set(x_82, 4, x_3); -if (lean_is_exclusive(x_70)) { - lean_ctor_release(x_70, 0); - lean_ctor_release(x_70, 1); - lean_ctor_release(x_70, 2); - lean_ctor_release(x_70, 3); - x_83 = x_70; +lean_inc(x_18); +lean_inc(x_68); +x_71 = lean_alloc_ctor(2, 3, 0); +lean_ctor_set(x_71, 0, x_68); +lean_ctor_set(x_71, 1, x_18); +lean_ctor_set(x_71, 2, x_69); +x_72 = lean_box(0); +lean_inc(x_68); +x_73 = l_Lean_mkNatLit(x_68); +x_74 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__3; +lean_inc(x_70); +lean_inc(x_1); +lean_inc(x_73); +x_75 = l_Lean_mkApp3(x_74, x_73, x_1, x_70); +x_76 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_76, 0, x_68); +lean_closure_set(x_76, 1, x_70); +lean_inc(x_65); +x_77 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13), 12, 5); +lean_closure_set(x_77, 0, x_65); +lean_closure_set(x_77, 1, x_72); +lean_closure_set(x_77, 2, x_1); +lean_closure_set(x_77, 3, x_73); +lean_closure_set(x_77, 4, x_2); +if (lean_is_exclusive(x_65)) { + lean_ctor_release(x_65, 0); + lean_ctor_release(x_65, 1); + lean_ctor_release(x_65, 2); + lean_ctor_release(x_65, 3); + x_78 = x_65; } else { - lean_dec_ref(x_70); - x_83 = lean_box(0); + lean_dec_ref(x_65); + x_78 = lean_box(0); } -x_84 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_84, 0, x_81); -lean_closure_set(x_84, 1, x_82); -if (lean_is_scalar(x_83)) { - x_85 = lean_alloc_ctor(0, 4, 0); +x_79 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_79, 0, x_76); +lean_closure_set(x_79, 1, x_77); +if (lean_is_scalar(x_78)) { + x_80 = lean_alloc_ctor(0, 4, 0); } else { - x_85 = x_83; -} -lean_ctor_set(x_85, 0, x_23); -lean_ctor_set(x_85, 1, x_76); -lean_ctor_set(x_85, 2, x_84); -lean_ctor_set(x_85, 3, x_80); -x_86 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_86, 0, x_85); -if (lean_is_scalar(x_72)) { - x_87 = lean_alloc_ctor(0, 2, 0); + x_80 = x_78; +} +lean_ctor_set(x_80, 0, x_18); +lean_ctor_set(x_80, 1, x_71); +lean_ctor_set(x_80, 2, x_79); +lean_ctor_set(x_80, 3, x_75); +x_81 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_81, 0, x_80); +if (lean_is_scalar(x_67)) { + x_82 = lean_alloc_ctor(0, 2, 0); } else { - x_87 = x_72; + x_82 = x_67; } -lean_ctor_set(x_87, 0, x_86); -lean_ctor_set(x_87, 1, x_71); -return x_87; +lean_ctor_set(x_82, 0, x_81); +lean_ctor_set(x_82, 1, x_66); +return x_82; } } } else { -uint8_t x_88; -lean_dec(x_23); -lean_dec(x_3); +uint8_t x_83; +lean_dec(x_18); lean_dec(x_2); -x_88 = !lean_is_exclusive(x_24); -if (x_88 == 0) +lean_dec(x_1); +x_83 = !lean_is_exclusive(x_19); +if (x_83 == 0) { -return x_24; +return x_19; } else { -lean_object* x_89; lean_object* x_90; lean_object* x_91; -x_89 = lean_ctor_get(x_24, 0); -x_90 = lean_ctor_get(x_24, 1); -lean_inc(x_90); -lean_inc(x_89); -lean_dec(x_24); -x_91 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_91, 0, x_89); -lean_ctor_set(x_91, 1, x_90); -return x_91; +lean_object* x_84; lean_object* x_85; lean_object* x_86; +x_84 = lean_ctor_get(x_19, 0); +x_85 = lean_ctor_get(x_19, 1); +lean_inc(x_85); +lean_inc(x_84); +lean_dec(x_19); +x_86 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_86, 0, x_84); +lean_ctor_set(x_86, 1, x_85); +return x_86; } } } } else { -uint8_t x_92; -lean_dec(x_8); +uint8_t x_87; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -5232,28 +4993,28 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_92 = !lean_is_exclusive(x_10); -if (x_92 == 0) +x_87 = !lean_is_exclusive(x_9); +if (x_87 == 0) { -return x_10; +return x_9; } else { -lean_object* x_93; lean_object* x_94; lean_object* x_95; -x_93 = lean_ctor_get(x_10, 0); -x_94 = lean_ctor_get(x_10, 1); -lean_inc(x_94); -lean_inc(x_93); -lean_dec(x_10); -x_95 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_95, 0, x_93); -lean_ctor_set(x_95, 1, x_94); -return x_95; +lean_object* x_88; lean_object* x_89; lean_object* x_90; +x_88 = lean_ctor_get(x_9, 0); +x_89 = lean_ctor_get(x_9, 1); +lean_inc(x_89); +lean_inc(x_88); +lean_dec(x_9); +x_90 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_90, 0, x_88); +lean_ctor_set(x_90, 1, x_89); +return x_90; } } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__15(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__15(lean_object* x_1) { _start: { lean_object* x_2; @@ -5262,7 +5023,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__1() { _start: { lean_object* x_1; @@ -5270,20 +5031,20 @@ x_1 = lean_mk_string_unchecked("arithShiftRightConst", 20, 20); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__1; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__1; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__3() { _start: { lean_object* x_1; @@ -5291,144 +5052,121 @@ x_1 = lean_mk_string_unchecked("arithShiftRight_congr", 21, 21); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__3; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__3; x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); return x_7; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__5() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__15), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__15), 1, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_10; -lean_inc(x_8); +lean_object* x_9; lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_10 = l_Lean_Meta_getNatValue_x3f(x_3, x_5, x_6, x_7, x_8, x_9); +lean_inc(x_4); +x_9 = l_Lean_Meta_getNatValue_x3f(x_2, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_9) == 0) +{ +lean_object* x_10; +x_10 = lean_ctor_get(x_9, 0); +lean_inc(x_10); if (lean_obj_tag(x_10) == 0) { -lean_object* x_11; -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -if (lean_obj_tag(x_11) == 0) +uint8_t x_11; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_11 = !lean_is_exclusive(x_9); +if (x_11 == 0) { lean_object* x_12; lean_object* x_13; -lean_dec(x_2); -x_12 = lean_ctor_get(x_10, 1); -lean_inc(x_12); -lean_dec(x_10); -x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_4, x_5, x_6, x_7, x_8, x_12); -if (lean_obj_tag(x_13) == 0) -{ -uint8_t x_14; -x_14 = !lean_is_exclusive(x_13); -if (x_14 == 0) -{ -return x_13; -} -else -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = lean_ctor_get(x_13, 0); -x_16 = lean_ctor_get(x_13, 1); -lean_inc(x_16); -lean_inc(x_15); -lean_dec(x_13); -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_15); -lean_ctor_set(x_17, 1, x_16); -return x_17; -} -} -else -{ -uint8_t x_18; -x_18 = !lean_is_exclusive(x_13); -if (x_18 == 0) -{ -return x_13; +x_12 = lean_ctor_get(x_9, 0); +lean_dec(x_12); +x_13 = lean_box(0); +lean_ctor_set(x_9, 0, x_13); +return x_9; } else { -lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_19 = lean_ctor_get(x_13, 0); -x_20 = lean_ctor_get(x_13, 1); -lean_inc(x_20); -lean_inc(x_19); -lean_dec(x_13); -x_21 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_21, 0, x_19); -lean_ctor_set(x_21, 1, x_20); -return x_21; -} +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_9, 1); +lean_inc(x_14); +lean_dec(x_9); +x_15 = lean_box(0); +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_16, 1, x_14); +return x_16; } } else { -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; -lean_dec(x_1); -x_22 = lean_ctor_get(x_10, 1); -lean_inc(x_22); +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_17 = lean_ctor_get(x_9, 1); +lean_inc(x_17); +lean_dec(x_9); +x_18 = lean_ctor_get(x_10, 0); +lean_inc(x_18); lean_dec(x_10); -x_23 = lean_ctor_get(x_11, 0); -lean_inc(x_23); -lean_dec(x_11); -x_24 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__5; -x_25 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__2; -x_26 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__4; -x_27 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftConstLikeReflection(x_23, x_2, x_24, x_25, x_26, x_4, x_5, x_6, x_7, x_8, x_22); -return x_27; +x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__5; +x_20 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__2; +x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__4; +x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftConstLikeReflection(x_18, x_1, x_19, x_20, x_21, x_3, x_4, x_5, x_6, x_7, x_17); +return x_22; } } else { -uint8_t x_28; -lean_dec(x_8); +uint8_t x_23; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_2); +lean_dec(x_3); lean_dec(x_1); -x_28 = !lean_is_exclusive(x_10); -if (x_28 == 0) +x_23 = !lean_is_exclusive(x_9); +if (x_23 == 0) { -return x_10; +return x_9; } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_10, 0); -x_30 = lean_ctor_get(x_10, 1); -lean_inc(x_30); -lean_inc(x_29); -lean_dec(x_10); -x_31 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_31, 0, x_29); -lean_ctor_set(x_31, 1, x_30); -return x_31; +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_9, 0); +x_25 = lean_ctor_get(x_9, 1); +lean_inc(x_25); +lean_inc(x_24); +lean_dec(x_9); +x_26 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_26, 0, x_24); +lean_ctor_set(x_26, 1, x_25); +return x_26; } } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__17(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__17(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; @@ -5440,7 +5178,7 @@ lean_ctor_set(x_5, 3, x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__18(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__18(lean_object* x_1) { _start: { lean_object* x_2; @@ -5449,7 +5187,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__1() { _start: { lean_object* x_1; @@ -5457,7 +5195,7 @@ x_1 = lean_mk_string_unchecked("shiftRight", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; @@ -5465,12 +5203,12 @@ x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__4; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__1; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__3() { _start: { lean_object* x_1; @@ -5478,29 +5216,29 @@ x_1 = lean_mk_string_unchecked("shiftRight_congr", 16, 16); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__3; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__3; x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); return x_7; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__5() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__17), 4, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__17), 4, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__6() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__6() { _start: { lean_object* x_1; @@ -5508,20 +5246,20 @@ x_1 = lean_mk_string_unchecked("shiftRightConst", 15, 15); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__7() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__6; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__6; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__8() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__8() { _start: { lean_object* x_1; @@ -5529,75 +5267,74 @@ x_1 = lean_mk_string_unchecked("shiftRightNat_congr", 19, 19); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__9() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__8; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__8; x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); return x_7; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__10() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__10() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__18), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__18), 1, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_11; -lean_inc(x_9); +lean_object* x_10; lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -lean_inc(x_2); -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_getNatOrBvValue_x3f(x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_inc(x_3); +lean_inc(x_1); +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_getNatOrBvValue_x3f(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_10) == 0) +{ +lean_object* x_11; +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); if (lean_obj_tag(x_11) == 0) { -lean_object* x_12; -x_12 = lean_ctor_get(x_11, 0); +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_12 = lean_ctor_get(x_10, 1); lean_inc(x_12); -if (lean_obj_tag(x_12) == 0) -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_13 = lean_ctor_get(x_11, 1); -lean_inc(x_13); -lean_dec(x_11); -x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__5; -x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__2; -x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__4; -x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection(x_1, x_2, x_4, x_3, x_14, x_15, x_16, x_5, x_6, x_7, x_8, x_9, x_13); -return x_17; +lean_dec(x_10); +x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__5; +x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__2; +x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__4; +x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection(x_1, x_3, x_2, x_13, x_14, x_15, x_4, x_5, x_6, x_7, x_8, x_12); +return x_16; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -lean_dec(x_12); -x_18 = lean_ctor_get(x_11, 1); -lean_inc(x_18); +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_dec(x_11); -x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__10; -x_20 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__7; -x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__9; -x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftConstReflection(x_1, x_2, x_4, x_3, x_19, x_20, x_21, x_5, x_6, x_7, x_8, x_9, x_18); -return x_22; +x_17 = lean_ctor_get(x_10, 1); +lean_inc(x_17); +lean_dec(x_10); +x_18 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__10; +x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__7; +x_20 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__9; +x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftConstReflection(x_1, x_3, x_2, x_18, x_19, x_20, x_4, x_5, x_6, x_7, x_8, x_17); +return x_21; } } else { -uint8_t x_23; -lean_dec(x_9); +uint8_t x_22; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -5606,28 +5343,28 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_23 = !lean_is_exclusive(x_11); -if (x_23 == 0) +x_22 = !lean_is_exclusive(x_10); +if (x_22 == 0) { -return x_11; +return x_10; } else -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_11, 0); -x_25 = lean_ctor_get(x_11, 1); -lean_inc(x_25); -lean_inc(x_24); -lean_dec(x_11); -x_26 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_26, 0, x_24); -lean_ctor_set(x_26, 1, x_25); -return x_26; +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_10, 0); +x_24 = lean_ctor_get(x_10, 1); +lean_inc(x_24); +lean_inc(x_23); +lean_dec(x_10); +x_25 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +return x_25; } } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__20(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__20(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; @@ -5639,7 +5376,7 @@ lean_ctor_set(x_5, 3, x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__21(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__21(lean_object* x_1) { _start: { lean_object* x_2; @@ -5648,7 +5385,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__1() { _start: { lean_object* x_1; @@ -5656,7 +5393,7 @@ x_1 = lean_mk_string_unchecked("shiftLeft", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; @@ -5664,12 +5401,12 @@ x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__4; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__1; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__3() { _start: { lean_object* x_1; @@ -5677,29 +5414,29 @@ x_1 = lean_mk_string_unchecked("shiftLeft_congr", 15, 15); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__3; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__3; x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); return x_7; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__5() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__20), 4, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__20), 4, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__6() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__6() { _start: { lean_object* x_1; @@ -5707,20 +5444,20 @@ x_1 = lean_mk_string_unchecked("shiftLeftConst", 14, 14); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__7() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__6; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__6; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__8() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__8() { _start: { lean_object* x_1; @@ -5728,75 +5465,74 @@ x_1 = lean_mk_string_unchecked("shiftLeftNat_congr", 18, 18); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__9() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__8; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__8; x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); return x_7; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__10() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__10() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__21), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__21), 1, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_11; -lean_inc(x_9); +lean_object* x_10; lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -lean_inc(x_2); -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_getNatOrBvValue_x3f(x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_inc(x_3); +lean_inc(x_1); +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_getNatOrBvValue_x3f(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_10) == 0) +{ +lean_object* x_11; +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); if (lean_obj_tag(x_11) == 0) { -lean_object* x_12; -x_12 = lean_ctor_get(x_11, 0); +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_12 = lean_ctor_get(x_10, 1); lean_inc(x_12); -if (lean_obj_tag(x_12) == 0) -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_13 = lean_ctor_get(x_11, 1); -lean_inc(x_13); -lean_dec(x_11); -x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__5; -x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__2; -x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__4; -x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection(x_1, x_2, x_4, x_3, x_14, x_15, x_16, x_5, x_6, x_7, x_8, x_9, x_13); -return x_17; +lean_dec(x_10); +x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__5; +x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__2; +x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__4; +x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection(x_1, x_3, x_2, x_13, x_14, x_15, x_4, x_5, x_6, x_7, x_8, x_12); +return x_16; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -lean_dec(x_12); -x_18 = lean_ctor_get(x_11, 1); -lean_inc(x_18); +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_dec(x_11); -x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__10; -x_20 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__7; -x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__9; -x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftConstReflection(x_1, x_2, x_4, x_3, x_19, x_20, x_21, x_5, x_6, x_7, x_8, x_9, x_18); -return x_22; +x_17 = lean_ctor_get(x_10, 1); +lean_inc(x_17); +lean_dec(x_10); +x_18 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__10; +x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__7; +x_20 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__9; +x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftConstReflection(x_1, x_3, x_2, x_18, x_19, x_20, x_4, x_5, x_6, x_7, x_8, x_17); +return x_21; } } else { -uint8_t x_23; -lean_dec(x_9); +uint8_t x_22; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -5805,28 +5541,28 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_23 = !lean_is_exclusive(x_11); -if (x_23 == 0) +x_22 = !lean_is_exclusive(x_10); +if (x_22 == 0) { -return x_11; +return x_10; } else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_11, 0); -x_25 = lean_ctor_get(x_11, 1); -lean_inc(x_25); +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_10, 0); +x_24 = lean_ctor_get(x_10, 1); lean_inc(x_24); -lean_dec(x_11); -x_26 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_26, 0, x_24); -lean_ctor_set(x_26, 1, x_25); -return x_26; +lean_inc(x_23); +lean_dec(x_10); +x_25 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +return x_25; } } } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__23___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__23___closed__1() { _start: { lean_object* x_1; @@ -5834,31 +5570,63 @@ x_1 = lean_mk_string_unchecked("not_congr", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__23___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__23___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__23___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__23___closed__1; x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__23(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__23(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; lean_object* x_9; lean_object* x_10; x_8 = lean_box(0); -x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__23___closed__2; +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__23___closed__2; x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_unaryReflection(x_1, x_8, x_9, x_2, x_3, x_4, x_5, x_6, x_7); return x_10; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__24___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__24___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("sdiv_congr", 10, 10); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__24___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__24___closed__1; +x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__24(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +uint8_t x_9; lean_object* x_10; lean_object* x_11; +x_9 = 7; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__24___closed__2; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection(x_1, x_2, x_9, x_10, x_3, x_4, x_5, x_6, x_7, x_8); +return x_11; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__25___closed__1() { _start: { lean_object* x_1; @@ -5866,31 +5634,31 @@ x_1 = lean_mk_string_unchecked("umod_congr", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__24___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__25___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__24___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__25___closed__1; x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__24(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__25(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { uint8_t x_9; lean_object* x_10; lean_object* x_11; x_9 = 6; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__24___closed__2; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__25___closed__2; x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection(x_1, x_2, x_9, x_10, x_3, x_4, x_5, x_6, x_7, x_8); return x_11; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__25___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__26___closed__1() { _start: { lean_object* x_1; @@ -5898,31 +5666,31 @@ x_1 = lean_mk_string_unchecked("udiv_congr", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__25___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__26___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__25___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__26___closed__1; x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__25(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__26(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { uint8_t x_9; lean_object* x_10; lean_object* x_11; x_9 = 5; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__25___closed__2; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__26___closed__2; x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection(x_1, x_2, x_9, x_10, x_3, x_4, x_5, x_6, x_7, x_8); return x_11; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__26___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__27___closed__1() { _start: { lean_object* x_1; @@ -5930,31 +5698,31 @@ x_1 = lean_mk_string_unchecked("mul_congr", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__26___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__27___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__26___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__27___closed__1; x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__26(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__27(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { uint8_t x_9; lean_object* x_10; lean_object* x_11; x_9 = 4; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__26___closed__2; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__27___closed__2; x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection(x_1, x_2, x_9, x_10, x_3, x_4, x_5, x_6, x_7, x_8); return x_11; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__27___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__28___closed__1() { _start: { lean_object* x_1; @@ -5962,31 +5730,31 @@ x_1 = lean_mk_string_unchecked("add_congr", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__27___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__28___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__27___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__28___closed__1; x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__27(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__28(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { uint8_t x_9; lean_object* x_10; lean_object* x_11; x_9 = 3; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__27___closed__2; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__28___closed__2; x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection(x_1, x_2, x_9, x_10, x_3, x_4, x_5, x_6, x_7, x_8); return x_11; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__28___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__29___closed__1() { _start: { lean_object* x_1; @@ -5994,31 +5762,31 @@ x_1 = lean_mk_string_unchecked("xor_congr", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__28___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__29___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__28___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__29___closed__1; x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__28(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__29(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { uint8_t x_9; lean_object* x_10; lean_object* x_11; x_9 = 2; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__28___closed__2; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__29___closed__2; x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection(x_1, x_2, x_9, x_10, x_3, x_4, x_5, x_6, x_7, x_8); return x_11; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__29___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__30___closed__1() { _start: { lean_object* x_1; @@ -6026,31 +5794,31 @@ x_1 = lean_mk_string_unchecked("or_congr", 8, 8); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__29___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__30___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__29___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__30___closed__1; x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__29(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__30(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { uint8_t x_9; lean_object* x_10; lean_object* x_11; x_9 = 1; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__29___closed__2; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__30___closed__2; x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection(x_1, x_2, x_9, x_10, x_3, x_4, x_5, x_6, x_7, x_8); return x_11; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__30___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__31___closed__1() { _start: { lean_object* x_1; @@ -6058,31 +5826,31 @@ x_1 = lean_mk_string_unchecked("and_congr", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__30___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__31___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__30___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__31___closed__1; x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__30(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__31(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { uint8_t x_9; lean_object* x_10; lean_object* x_11; x_9 = 0; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__30___closed__2; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__31___closed__2; x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection(x_1, x_2, x_9, x_10, x_3, x_4, x_5, x_6, x_7, x_8); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__31(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__32(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; @@ -6090,137 +5858,209 @@ x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goBvLit(x_1, x_3, x_ return x_9; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__32(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__1() { _start: { -lean_object* x_9; -x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_3, x_4, x_5, x_6, x_7, x_8); -return x_9; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___boxed), 8, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___boxed), 8, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6), 9, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___boxed), 8, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10), 8, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12), 8, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__7() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14), 8, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__8() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___boxed), 8, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__9() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19), 9, 0); +return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__10() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10), 8, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22), 9, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__11() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__23), 7, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__23), 7, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__12() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__24), 8, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__24), 8, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__13() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__25), 8, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__25), 8, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__14() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__26), 8, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__26), 8, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__6() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__15() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__27), 8, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__27), 8, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__7() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__16() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__28), 8, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__28), 8, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__8() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__17() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__29), 8, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__29), 8, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__9() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__18() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__30), 8, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__30), 8, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__10() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__19() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__31), 8, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__20() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__2; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__2; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__11() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__21() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__1; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__12() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__22() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__1; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__13() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__23() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__1; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__14() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__24() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__1; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__15() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__25() { _start: { lean_object* x_1; @@ -6228,17 +6068,17 @@ x_1 = lean_mk_string_unchecked("sshiftRight", 11, 11); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__16() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__26() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__15; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__25; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__17() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__27() { _start: { lean_object* x_1; @@ -6246,7 +6086,7 @@ x_1 = lean_mk_string_unchecked("Complement", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__18() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__28() { _start: { lean_object* x_1; @@ -6254,17 +6094,35 @@ x_1 = lean_mk_string_unchecked("complement", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__19() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__29() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__27; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__28; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__30() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("sdiv", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__31() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__17; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__18; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__30; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__20() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__32() { _start: { lean_object* x_1; @@ -6272,17 +6130,17 @@ x_1 = lean_mk_string_unchecked("extractLsb'", 11, 11); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__21() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__33() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__20; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__32; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__22() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__34() { _start: { lean_object* x_1; @@ -6290,7 +6148,7 @@ x_1 = lean_mk_string_unchecked("HAppend", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__23() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__35() { _start: { lean_object* x_1; @@ -6298,17 +6156,17 @@ x_1 = lean_mk_string_unchecked("hAppend", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__24() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__36() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__22; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__23; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__34; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__35; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__25() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__37() { _start: { lean_object* x_1; @@ -6316,7 +6174,7 @@ x_1 = lean_mk_string_unchecked("HShiftRight", 11, 11); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__26() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__38() { _start: { lean_object* x_1; @@ -6324,17 +6182,17 @@ x_1 = lean_mk_string_unchecked("hShiftRight", 11, 11); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__27() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__39() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__25; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__26; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__37; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__38; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__28() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__40() { _start: { lean_object* x_1; @@ -6342,7 +6200,7 @@ x_1 = lean_mk_string_unchecked("HShiftLeft", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__29() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__41() { _start: { lean_object* x_1; @@ -6350,17 +6208,17 @@ x_1 = lean_mk_string_unchecked("hShiftLeft", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__30() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__42() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__28; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__29; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__40; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__41; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__31() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__43() { _start: { lean_object* x_1; @@ -6368,7 +6226,7 @@ x_1 = lean_mk_string_unchecked("HMod", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__32() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__44() { _start: { lean_object* x_1; @@ -6376,17 +6234,17 @@ x_1 = lean_mk_string_unchecked("hMod", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__33() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__45() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__31; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__32; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__43; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__44; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__34() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__46() { _start: { lean_object* x_1; @@ -6394,7 +6252,7 @@ x_1 = lean_mk_string_unchecked("HDiv", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__35() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__47() { _start: { lean_object* x_1; @@ -6402,17 +6260,17 @@ x_1 = lean_mk_string_unchecked("hDiv", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__36() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__48() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__34; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__35; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__46; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__47; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__37() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__49() { _start: { lean_object* x_1; @@ -6420,7 +6278,7 @@ x_1 = lean_mk_string_unchecked("HMul", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__38() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__50() { _start: { lean_object* x_1; @@ -6428,17 +6286,17 @@ x_1 = lean_mk_string_unchecked("hMul", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__39() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__51() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__37; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__38; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__49; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__50; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__40() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__52() { _start: { lean_object* x_1; @@ -6446,7 +6304,7 @@ x_1 = lean_mk_string_unchecked("HAdd", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__41() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__53() { _start: { lean_object* x_1; @@ -6454,17 +6312,17 @@ x_1 = lean_mk_string_unchecked("hAdd", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__42() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__54() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__40; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__41; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__52; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__53; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__43() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__55() { _start: { lean_object* x_1; @@ -6472,7 +6330,7 @@ x_1 = lean_mk_string_unchecked("HXor", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__44() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__56() { _start: { lean_object* x_1; @@ -6480,17 +6338,17 @@ x_1 = lean_mk_string_unchecked("hXor", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__45() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__57() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__43; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__44; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__55; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__56; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__46() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__58() { _start: { lean_object* x_1; @@ -6498,7 +6356,7 @@ x_1 = lean_mk_string_unchecked("HOr", 3, 3); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__47() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__59() { _start: { lean_object* x_1; @@ -6506,17 +6364,17 @@ x_1 = lean_mk_string_unchecked("hOr", 3, 3); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__48() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__60() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__46; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__47; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__58; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__59; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__49() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__61() { _start: { lean_object* x_1; @@ -6524,7 +6382,7 @@ x_1 = lean_mk_string_unchecked("HAnd", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__50() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__62() { _start: { lean_object* x_1; @@ -6532,20 +6390,20 @@ x_1 = lean_mk_string_unchecked("hAnd", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__51() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__63() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__49; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__50; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__61; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__62; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; lean_inc(x_1); x_8 = l_Lean_Meta_instantiateMVarsIfMVarApp(x_1, x_3, x_4, x_5, x_6, x_7); x_9 = lean_ctor_get(x_8, 0); @@ -6553,383 +6411,405 @@ lean_inc(x_9); x_10 = lean_ctor_get(x_8, 1); lean_inc(x_10); lean_dec(x_8); -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__1; -x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__2; -x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__3; -x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__4; -x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__5; -x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__6; -x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__7; -x_18 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__8; -x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__9; -x_20 = l_Lean_Expr_cleanupAnnotations(x_9); -x_21 = l_Lean_Expr_isApp(x_20); -if (x_21 == 0) +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__1; +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__2; +x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__3; +x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__4; +x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__5; +x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__6; +x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__7; +x_18 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__8; +x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__9; +x_20 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__10; +x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__11; +x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__12; +x_23 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__13; +x_24 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__14; +x_25 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__15; +x_26 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__16; +x_27 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__17; +x_28 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__18; +x_29 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__19; +x_30 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_getNatOrBvValue_x3f___closed__1; +x_31 = l_Lean_Expr_cleanupAnnotations(x_9); +x_32 = l_Lean_Expr_isApp(x_31); +if (x_32 == 0) { -lean_object* x_22; -lean_dec(x_20); -x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_2, x_3, x_4, x_5, x_6, x_10); -return x_22; +lean_object* x_33; lean_object* x_34; +lean_dec(x_31); +lean_dec(x_1); +x_33 = lean_box(0); +x_34 = lean_apply_7(x_30, x_33, x_2, x_3, x_4, x_5, x_6, x_10); +return x_34; } else { -lean_object* x_23; lean_object* x_24; uint8_t x_25; -x_23 = l_Lean_Expr_appArg(x_20, lean_box(0)); -x_24 = l_Lean_Expr_appFnCleanup(x_20, lean_box(0)); -x_25 = l_Lean_Expr_isApp(x_24); -if (x_25 == 0) +lean_object* x_35; lean_object* x_36; uint8_t x_37; +x_35 = l_Lean_Expr_appArg(x_31, lean_box(0)); +x_36 = l_Lean_Expr_appFnCleanup(x_31, lean_box(0)); +x_37 = l_Lean_Expr_isApp(x_36); +if (x_37 == 0) { -lean_object* x_26; -lean_dec(x_24); -lean_dec(x_23); -x_26 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_2, x_3, x_4, x_5, x_6, x_10); -return x_26; +lean_object* x_38; lean_object* x_39; +lean_dec(x_36); +lean_dec(x_35); +lean_dec(x_1); +x_38 = lean_box(0); +x_39 = lean_apply_7(x_30, x_38, x_2, x_3, x_4, x_5, x_6, x_10); +return x_39; } else { -lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; -x_27 = l_Lean_Expr_appArg(x_24, lean_box(0)); -x_28 = l_Lean_Expr_appFnCleanup(x_24, lean_box(0)); -x_29 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goBvLit___closed__5; -x_30 = l_Lean_Expr_isConstOf(x_28, x_29); -if (x_30 == 0) +lean_object* x_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; +x_40 = l_Lean_Expr_appArg(x_36, lean_box(0)); +x_41 = l_Lean_Expr_appFnCleanup(x_36, lean_box(0)); +x_42 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goBvLit___closed__5; +x_43 = l_Lean_Expr_isConstOf(x_41, x_42); +if (x_43 == 0) { -uint8_t x_31; -x_31 = l_Lean_Expr_isApp(x_28); -if (x_31 == 0) +uint8_t x_44; +lean_dec(x_1); +x_44 = l_Lean_Expr_isApp(x_41); +if (x_44 == 0) { -lean_object* x_32; -lean_dec(x_28); -lean_dec(x_27); -lean_dec(x_23); -x_32 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_2, x_3, x_4, x_5, x_6, x_10); -return x_32; +lean_object* x_45; lean_object* x_46; +lean_dec(x_41); +lean_dec(x_40); +lean_dec(x_35); +x_45 = lean_box(0); +x_46 = lean_apply_7(x_30, x_45, x_2, x_3, x_4, x_5, x_6, x_10); +return x_46; } else { -lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; -x_33 = l_Lean_Expr_appArg(x_28, lean_box(0)); -x_34 = l_Lean_Expr_appFnCleanup(x_28, lean_box(0)); -x_35 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__10; -x_36 = l_Lean_Expr_isConstOf(x_34, x_35); -if (x_36 == 0) +lean_object* x_47; lean_object* x_48; lean_object* x_49; uint8_t x_50; +x_47 = l_Lean_Expr_appArg(x_41, lean_box(0)); +x_48 = l_Lean_Expr_appFnCleanup(x_41, lean_box(0)); +x_49 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__20; +x_50 = l_Lean_Expr_isConstOf(x_48, x_49); +if (x_50 == 0) +{ +lean_object* x_51; uint8_t x_52; +x_51 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__21; +x_52 = l_Lean_Expr_isConstOf(x_48, x_51); +if (x_52 == 0) { -lean_object* x_37; uint8_t x_38; -x_37 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__11; -x_38 = l_Lean_Expr_isConstOf(x_34, x_37); -if (x_38 == 0) +lean_object* x_53; uint8_t x_54; +x_53 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__22; +x_54 = l_Lean_Expr_isConstOf(x_48, x_53); +if (x_54 == 0) { -lean_object* x_39; uint8_t x_40; -x_39 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__12; -x_40 = l_Lean_Expr_isConstOf(x_34, x_39); -if (x_40 == 0) +lean_object* x_55; uint8_t x_56; +x_55 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__23; +x_56 = l_Lean_Expr_isConstOf(x_48, x_55); +if (x_56 == 0) { -lean_object* x_41; uint8_t x_42; -x_41 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__13; -x_42 = l_Lean_Expr_isConstOf(x_34, x_41); -if (x_42 == 0) +lean_object* x_57; uint8_t x_58; +x_57 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__24; +x_58 = l_Lean_Expr_isConstOf(x_48, x_57); +if (x_58 == 0) { -lean_object* x_43; uint8_t x_44; -x_43 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__14; -x_44 = l_Lean_Expr_isConstOf(x_34, x_43); -if (x_44 == 0) +lean_object* x_59; uint8_t x_60; +x_59 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__26; +x_60 = l_Lean_Expr_isConstOf(x_48, x_59); +if (x_60 == 0) { -lean_object* x_45; uint8_t x_46; -x_45 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__16; -x_46 = l_Lean_Expr_isConstOf(x_34, x_45); -if (x_46 == 0) +lean_object* x_61; uint8_t x_62; +x_61 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__29; +x_62 = l_Lean_Expr_isConstOf(x_48, x_61); +if (x_62 == 0) { -lean_object* x_47; uint8_t x_48; -x_47 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__19; -x_48 = l_Lean_Expr_isConstOf(x_34, x_47); -if (x_48 == 0) +lean_object* x_63; uint8_t x_64; +x_63 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__31; +x_64 = l_Lean_Expr_isConstOf(x_48, x_63); +if (x_64 == 0) { -uint8_t x_49; -x_49 = l_Lean_Expr_isApp(x_34); -if (x_49 == 0) +uint8_t x_65; +x_65 = l_Lean_Expr_isApp(x_48); +if (x_65 == 0) { -lean_object* x_50; -lean_dec(x_34); -lean_dec(x_33); -lean_dec(x_27); -lean_dec(x_23); -x_50 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_2, x_3, x_4, x_5, x_6, x_10); -return x_50; +lean_object* x_66; lean_object* x_67; +lean_dec(x_48); +lean_dec(x_47); +lean_dec(x_40); +lean_dec(x_35); +x_66 = lean_box(0); +x_67 = lean_apply_7(x_30, x_66, x_2, x_3, x_4, x_5, x_6, x_10); +return x_67; } else { -lean_object* x_51; lean_object* x_52; uint8_t x_53; -x_51 = l_Lean_Expr_appFnCleanup(x_34, lean_box(0)); -x_52 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__21; -x_53 = l_Lean_Expr_isConstOf(x_51, x_52); -if (x_53 == 0) +lean_object* x_68; lean_object* x_69; uint8_t x_70; +x_68 = l_Lean_Expr_appFnCleanup(x_48, lean_box(0)); +x_69 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__33; +x_70 = l_Lean_Expr_isConstOf(x_68, x_69); +if (x_70 == 0) { -uint8_t x_54; -lean_dec(x_33); -x_54 = l_Lean_Expr_isApp(x_51); -if (x_54 == 0) +uint8_t x_71; +lean_dec(x_47); +x_71 = l_Lean_Expr_isApp(x_68); +if (x_71 == 0) { -lean_object* x_55; -lean_dec(x_51); -lean_dec(x_27); -lean_dec(x_23); -x_55 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_2, x_3, x_4, x_5, x_6, x_10); -return x_55; +lean_object* x_72; lean_object* x_73; +lean_dec(x_68); +lean_dec(x_40); +lean_dec(x_35); +x_72 = lean_box(0); +x_73 = lean_apply_7(x_30, x_72, x_2, x_3, x_4, x_5, x_6, x_10); +return x_73; } else { -lean_object* x_56; lean_object* x_57; uint8_t x_58; -x_56 = l_Lean_Expr_appArg(x_51, lean_box(0)); -x_57 = l_Lean_Expr_appFnCleanup(x_51, lean_box(0)); -x_58 = l_Lean_Expr_isApp(x_57); -if (x_58 == 0) +lean_object* x_74; lean_object* x_75; uint8_t x_76; +x_74 = l_Lean_Expr_appArg(x_68, lean_box(0)); +x_75 = l_Lean_Expr_appFnCleanup(x_68, lean_box(0)); +x_76 = l_Lean_Expr_isApp(x_75); +if (x_76 == 0) { -lean_object* x_59; -lean_dec(x_57); -lean_dec(x_56); -lean_dec(x_27); -lean_dec(x_23); -x_59 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_2, x_3, x_4, x_5, x_6, x_10); -return x_59; +lean_object* x_77; lean_object* x_78; +lean_dec(x_75); +lean_dec(x_74); +lean_dec(x_40); +lean_dec(x_35); +x_77 = lean_box(0); +x_78 = lean_apply_7(x_30, x_77, x_2, x_3, x_4, x_5, x_6, x_10); +return x_78; } else { -lean_object* x_60; lean_object* x_61; uint8_t x_62; -x_60 = l_Lean_Expr_appFnCleanup(x_57, lean_box(0)); -x_61 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__24; -x_62 = l_Lean_Expr_isConstOf(x_60, x_61); -if (x_62 == 0) -{ -lean_object* x_63; uint8_t x_64; -x_63 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__27; -x_64 = l_Lean_Expr_isConstOf(x_60, x_63); -if (x_64 == 0) -{ -lean_object* x_65; uint8_t x_66; -x_65 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__30; -x_66 = l_Lean_Expr_isConstOf(x_60, x_65); -if (x_66 == 0) -{ -lean_object* x_67; uint8_t x_68; -lean_dec(x_56); -x_67 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__33; -x_68 = l_Lean_Expr_isConstOf(x_60, x_67); -if (x_68 == 0) -{ -lean_object* x_69; uint8_t x_70; -x_69 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__36; -x_70 = l_Lean_Expr_isConstOf(x_60, x_69); -if (x_70 == 0) +lean_object* x_79; lean_object* x_80; uint8_t x_81; +x_79 = l_Lean_Expr_appFnCleanup(x_75, lean_box(0)); +x_80 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__36; +x_81 = l_Lean_Expr_isConstOf(x_79, x_80); +if (x_81 == 0) { -lean_object* x_71; uint8_t x_72; -x_71 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__39; -x_72 = l_Lean_Expr_isConstOf(x_60, x_71); -if (x_72 == 0) +lean_object* x_82; uint8_t x_83; +x_82 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__39; +x_83 = l_Lean_Expr_isConstOf(x_79, x_82); +if (x_83 == 0) { -lean_object* x_73; uint8_t x_74; -x_73 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__42; -x_74 = l_Lean_Expr_isConstOf(x_60, x_73); -if (x_74 == 0) +lean_object* x_84; uint8_t x_85; +x_84 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__42; +x_85 = l_Lean_Expr_isConstOf(x_79, x_84); +if (x_85 == 0) { -lean_object* x_75; uint8_t x_76; -x_75 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__45; -x_76 = l_Lean_Expr_isConstOf(x_60, x_75); -if (x_76 == 0) +lean_object* x_86; uint8_t x_87; +lean_dec(x_74); +x_86 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__45; +x_87 = l_Lean_Expr_isConstOf(x_79, x_86); +if (x_87 == 0) { -lean_object* x_77; uint8_t x_78; -x_77 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__48; -x_78 = l_Lean_Expr_isConstOf(x_60, x_77); -if (x_78 == 0) +lean_object* x_88; uint8_t x_89; +x_88 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__48; +x_89 = l_Lean_Expr_isConstOf(x_79, x_88); +if (x_89 == 0) +{ +lean_object* x_90; uint8_t x_91; +x_90 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__51; +x_91 = l_Lean_Expr_isConstOf(x_79, x_90); +if (x_91 == 0) +{ +lean_object* x_92; uint8_t x_93; +x_92 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__54; +x_93 = l_Lean_Expr_isConstOf(x_79, x_92); +if (x_93 == 0) +{ +lean_object* x_94; uint8_t x_95; +x_94 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__57; +x_95 = l_Lean_Expr_isConstOf(x_79, x_94); +if (x_95 == 0) +{ +lean_object* x_96; uint8_t x_97; +x_96 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__60; +x_97 = l_Lean_Expr_isConstOf(x_79, x_96); +if (x_97 == 0) { -lean_object* x_79; uint8_t x_80; -x_79 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__51; -x_80 = l_Lean_Expr_isConstOf(x_60, x_79); -lean_dec(x_60); -if (x_80 == 0) +lean_object* x_98; uint8_t x_99; +x_98 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__63; +x_99 = l_Lean_Expr_isConstOf(x_79, x_98); +lean_dec(x_79); +if (x_99 == 0) { -lean_object* x_81; -lean_dec(x_27); -lean_dec(x_23); -x_81 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_2, x_3, x_4, x_5, x_6, x_10); -return x_81; +lean_object* x_100; lean_object* x_101; +lean_dec(x_40); +lean_dec(x_35); +x_100 = lean_box(0); +x_101 = lean_apply_7(x_30, x_100, x_2, x_3, x_4, x_5, x_6, x_10); +return x_101; } else { -lean_object* x_82; -lean_dec(x_1); -x_82 = lean_apply_8(x_19, x_27, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_82; +lean_object* x_102; +x_102 = lean_apply_8(x_29, x_40, x_35, x_2, x_3, x_4, x_5, x_6, x_10); +return x_102; } } else { -lean_object* x_83; -lean_dec(x_60); -lean_dec(x_1); -x_83 = lean_apply_8(x_18, x_27, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_83; +lean_object* x_103; +lean_dec(x_79); +x_103 = lean_apply_8(x_28, x_40, x_35, x_2, x_3, x_4, x_5, x_6, x_10); +return x_103; } } else { -lean_object* x_84; -lean_dec(x_60); -lean_dec(x_1); -x_84 = lean_apply_8(x_17, x_27, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_84; +lean_object* x_104; +lean_dec(x_79); +x_104 = lean_apply_8(x_27, x_40, x_35, x_2, x_3, x_4, x_5, x_6, x_10); +return x_104; } } else { -lean_object* x_85; -lean_dec(x_60); -lean_dec(x_1); -x_85 = lean_apply_8(x_16, x_27, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_85; +lean_object* x_105; +lean_dec(x_79); +x_105 = lean_apply_8(x_26, x_40, x_35, x_2, x_3, x_4, x_5, x_6, x_10); +return x_105; } } else { -lean_object* x_86; -lean_dec(x_60); -lean_dec(x_1); -x_86 = lean_apply_8(x_15, x_27, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_86; +lean_object* x_106; +lean_dec(x_79); +x_106 = lean_apply_8(x_25, x_40, x_35, x_2, x_3, x_4, x_5, x_6, x_10); +return x_106; } } else { -lean_object* x_87; -lean_dec(x_60); -lean_dec(x_1); -x_87 = lean_apply_8(x_14, x_27, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_87; +lean_object* x_107; +lean_dec(x_79); +x_107 = lean_apply_8(x_24, x_40, x_35, x_2, x_3, x_4, x_5, x_6, x_10); +return x_107; } } else { -lean_object* x_88; -lean_dec(x_60); -lean_dec(x_1); -x_88 = lean_apply_8(x_13, x_27, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_88; +lean_object* x_108; +lean_dec(x_79); +x_108 = lean_apply_8(x_23, x_40, x_35, x_2, x_3, x_4, x_5, x_6, x_10); +return x_108; } } else { -lean_object* x_89; -lean_dec(x_60); -x_89 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22(x_1, x_56, x_27, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_89; +lean_object* x_109; +lean_dec(x_79); +x_109 = lean_apply_9(x_20, x_74, x_40, x_35, x_2, x_3, x_4, x_5, x_6, x_10); +return x_109; } } else { -lean_object* x_90; -lean_dec(x_60); -x_90 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19(x_1, x_56, x_27, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_90; +lean_object* x_110; +lean_dec(x_79); +x_110 = lean_apply_9(x_19, x_74, x_40, x_35, x_2, x_3, x_4, x_5, x_6, x_10); +return x_110; } } else { -lean_object* x_91; -lean_dec(x_60); -lean_dec(x_56); -lean_dec(x_1); -x_91 = lean_apply_8(x_11, x_27, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_91; +lean_object* x_111; +lean_dec(x_79); +lean_dec(x_74); +x_111 = lean_apply_8(x_15, x_40, x_35, x_2, x_3, x_4, x_5, x_6, x_10); +return x_111; } } } } else { -lean_object* x_92; -lean_dec(x_51); -x_92 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6(x_1, x_33, x_27, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_92; +lean_object* x_112; +lean_dec(x_68); +x_112 = lean_apply_9(x_13, x_47, x_40, x_35, x_2, x_3, x_4, x_5, x_6, x_10); +return x_112; } } } else { -lean_object* x_93; -lean_dec(x_34); -lean_dec(x_33); -lean_dec(x_27); -lean_dec(x_1); -x_93 = lean_apply_7(x_12, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_93; +lean_object* x_113; +lean_dec(x_48); +lean_dec(x_47); +x_113 = lean_apply_8(x_22, x_40, x_35, x_2, x_3, x_4, x_5, x_6, x_10); +return x_113; } } else { -lean_object* x_94; -lean_dec(x_34); -lean_dec(x_33); -x_94 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16(x_1, x_27, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -lean_dec(x_23); -return x_94; +lean_object* x_114; +lean_dec(x_48); +lean_dec(x_47); +lean_dec(x_40); +x_114 = lean_apply_7(x_21, x_35, x_2, x_3, x_4, x_5, x_6, x_10); +return x_114; } } else { -lean_object* x_95; -lean_dec(x_34); -lean_dec(x_33); -x_95 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14(x_1, x_27, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_95; +lean_object* x_115; +lean_dec(x_48); +lean_dec(x_47); +x_115 = lean_apply_8(x_18, x_40, x_35, x_2, x_3, x_4, x_5, x_6, x_10); +return x_115; } } else { -lean_object* x_96; -lean_dec(x_34); -lean_dec(x_33); -x_96 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12(x_1, x_27, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_96; +lean_object* x_116; +lean_dec(x_48); +lean_dec(x_47); +x_116 = lean_apply_8(x_17, x_40, x_35, x_2, x_3, x_4, x_5, x_6, x_10); +return x_116; } } else { -lean_object* x_97; -lean_dec(x_34); -lean_dec(x_33); -x_97 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8(x_1, x_27, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -lean_dec(x_27); -return x_97; +lean_object* x_117; +lean_dec(x_48); +lean_dec(x_47); +x_117 = lean_apply_8(x_16, x_40, x_35, x_2, x_3, x_4, x_5, x_6, x_10); +return x_117; } } else { -lean_object* x_98; -lean_dec(x_34); -lean_dec(x_33); -x_98 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4(x_1, x_27, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -lean_dec(x_23); -return x_98; +lean_object* x_118; +lean_dec(x_48); +lean_dec(x_47); +x_118 = lean_apply_8(x_14, x_40, x_35, x_2, x_3, x_4, x_5, x_6, x_10); +return x_118; } } else { -lean_object* x_99; -lean_dec(x_34); -lean_dec(x_33); -x_99 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2(x_1, x_27, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -lean_dec(x_23); -return x_99; +lean_object* x_119; +lean_dec(x_48); +lean_dec(x_47); +x_119 = lean_apply_8(x_12, x_40, x_35, x_2, x_3, x_4, x_5, x_6, x_10); +return x_119; +} +} +else +{ +lean_object* x_120; +lean_dec(x_48); +lean_dec(x_47); +x_120 = lean_apply_8(x_11, x_40, x_35, x_2, x_3, x_4, x_5, x_6, x_10); +return x_120; } } } else { -lean_object* x_100; -lean_dec(x_28); -lean_dec(x_27); -lean_dec(x_23); -x_100 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goBvLit(x_1, x_2, x_3, x_4, x_5, x_6, x_10); -return x_100; +lean_object* x_121; +lean_dec(x_41); +lean_dec(x_40); +lean_dec(x_35); +x_121 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goBvLit(x_1, x_2, x_3, x_4, x_5, x_6, x_10); +return x_121; } } } @@ -7191,6 +7071,29 @@ x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__26() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__4; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__30; +x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__27() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__26; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { @@ -7201,7 +7104,7 @@ lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_1); -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofOrAtom(x_1, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(x_1, x_5, x_6, x_7, x_8, x_9, x_10); if (lean_obj_tag(x_11) == 0) { lean_object* x_12; @@ -7251,7 +7154,7 @@ x_20 = lean_ctor_get(x_12, 0); lean_inc(x_20); lean_dec(x_12); lean_inc(x_2); -x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofOrAtom(x_2, x_5, x_6, x_7, x_8, x_9, x_19); +x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(x_2, x_5, x_6, x_7, x_8, x_9, x_19); if (lean_obj_tag(x_21) == 0) { lean_object* x_22; @@ -7420,13 +7323,20 @@ x_61 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___ x_49 = x_61; goto block_55; } -default: +case 6: { lean_object* x_62; x_62 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__25; x_49 = x_62; goto block_55; } +default: +{ +lean_object* x_63; +x_63 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__27; +x_49 = x_63; +goto block_55; +} } block_55: { @@ -7462,35 +7372,35 @@ return x_54; } else { -uint8_t x_63; +uint8_t x_64; lean_dec(x_20); lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_63 = !lean_is_exclusive(x_21); -if (x_63 == 0) +x_64 = !lean_is_exclusive(x_21); +if (x_64 == 0) { return x_21; } else { -lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_64 = lean_ctor_get(x_21, 0); -x_65 = lean_ctor_get(x_21, 1); +lean_object* x_65; lean_object* x_66; lean_object* x_67; +x_65 = lean_ctor_get(x_21, 0); +x_66 = lean_ctor_get(x_21, 1); +lean_inc(x_66); lean_inc(x_65); -lean_inc(x_64); lean_dec(x_21); -x_66 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_66, 0, x_64); -lean_ctor_set(x_66, 1, x_65); -return x_66; +x_67 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_67, 0, x_65); +lean_ctor_set(x_67, 1, x_66); +return x_67; } } } } else { -uint8_t x_67; +uint8_t x_68; lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -7499,23 +7409,138 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_67 = !lean_is_exclusive(x_11); -if (x_67 == 0) +x_68 = !lean_is_exclusive(x_11); +if (x_68 == 0) { return x_11; } else { -lean_object* x_68; lean_object* x_69; lean_object* x_70; -x_68 = lean_ctor_get(x_11, 0); -x_69 = lean_ctor_get(x_11, 1); +lean_object* x_69; lean_object* x_70; lean_object* x_71; +x_69 = lean_ctor_get(x_11, 0); +x_70 = lean_ctor_get(x_11, 1); +lean_inc(x_70); lean_inc(x_69); -lean_inc(x_68); lean_dec(x_11); -x_70 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_70, 0, x_68); -lean_ctor_set(x_70, 1, x_69); -return x_70; +x_71 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_71, 0, x_69); +lean_ctor_set(x_71, 1, x_70); +return x_71; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +if (lean_obj_tag(x_8) == 0) +{ +lean_object* x_9; +x_9 = lean_ctor_get(x_8, 0); +lean_inc(x_9); +if (lean_obj_tag(x_9) == 0) +{ +lean_object* x_10; lean_object* x_11; +x_10 = lean_ctor_get(x_8, 1); +lean_inc(x_10); +lean_dec(x_8); +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom(x_1, x_2, x_3, x_4, x_5, x_6, x_10); +return x_11; +} +else +{ +uint8_t x_12; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_12 = !lean_is_exclusive(x_8); +if (x_12 == 0) +{ +lean_object* x_13; uint8_t x_14; +x_13 = lean_ctor_get(x_8, 0); +lean_dec(x_13); +x_14 = !lean_is_exclusive(x_9); +if (x_14 == 0) +{ +return x_8; +} +else +{ +lean_object* x_15; lean_object* x_16; +x_15 = lean_ctor_get(x_9, 0); +lean_inc(x_15); +lean_dec(x_9); +x_16 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_8, 0, x_16); +return x_8; +} +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_17 = lean_ctor_get(x_8, 1); +lean_inc(x_17); +lean_dec(x_8); +x_18 = lean_ctor_get(x_9, 0); +lean_inc(x_18); +if (lean_is_exclusive(x_9)) { + lean_ctor_release(x_9, 0); + x_19 = x_9; +} else { + lean_dec_ref(x_9); + x_19 = lean_box(0); +} +if (lean_is_scalar(x_19)) { + x_20 = lean_alloc_ctor(1, 1, 0); +} else { + x_20 = x_19; +} +lean_ctor_set(x_20, 0, x_18); +x_21 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_21, 0, x_20); +lean_ctor_set(x_21, 1, x_17); +return x_21; +} +} +} +else +{ +uint8_t x_22; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_22 = !lean_is_exclusive(x_8); +if (x_22 == 0) +{ +return x_8; +} +else +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_8, 0); +x_24 = lean_ctor_get(x_8, 1); +lean_inc(x_24); +lean_inc(x_23); +lean_dec(x_8); +x_25 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +return x_25; } } } @@ -7566,7 +7591,7 @@ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_obj x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__1; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__1; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_unaryReflection___closed__4; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -7587,7 +7612,7 @@ static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__7; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__7; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } @@ -7597,7 +7622,7 @@ static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__7; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__7; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } @@ -7607,7 +7632,7 @@ static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__2; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__2; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } @@ -7617,7 +7642,7 @@ static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__3; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__3; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } @@ -7627,7 +7652,7 @@ static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__2; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__2; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } @@ -7637,7 +7662,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_u { lean_object* x_10; lean_inc(x_1); -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofOrAtom(x_1, x_4, x_5, x_6, x_7, x_8, x_9); +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(x_1, x_4, x_5, x_6, x_7, x_8, x_9); if (lean_obj_tag(x_10) == 0) { lean_object* x_11; @@ -8392,7 +8417,7 @@ lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_1); -x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of(x_1, x_7, x_8, x_9, x_10, x_11, x_12); +x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(x_1, x_7, x_8, x_9, x_10, x_11, x_12); if (lean_obj_tag(x_13) == 0) { lean_object* x_14; @@ -8444,7 +8469,7 @@ x_22 = lean_ctor_get(x_14, 0); lean_inc(x_22); lean_dec(x_14); lean_inc(x_2); -x_23 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of(x_2, x_7, x_8, x_9, x_10, x_11, x_21); +x_23 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(x_2, x_7, x_8, x_9, x_10, x_11, x_21); if (lean_obj_tag(x_23) == 0) { lean_object* x_24; @@ -8765,80 +8790,30 @@ return x_104; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; -x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_3, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_9) == 0) -{ -uint8_t x_10; -x_10 = !lean_is_exclusive(x_9); -if (x_10 == 0) -{ -return x_9; -} -else -{ -lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_11 = lean_ctor_get(x_9, 0); -x_12 = lean_ctor_get(x_9, 1); -lean_inc(x_12); -lean_inc(x_11); -lean_dec(x_9); -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_11); -lean_ctor_set(x_13, 1, x_12); -return x_13; -} -} -else -{ -uint8_t x_14; -x_14 = !lean_is_exclusive(x_9); -if (x_14 == 0) -{ -return x_9; -} -else -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = lean_ctor_get(x_9, 0); -x_16 = lean_ctor_get(x_9, 1); -lean_inc(x_16); -lean_inc(x_15); -lean_dec(x_9); -x_17 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_17, 0, x_15); -lean_ctor_set(x_17, 1, x_16); -return x_17; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; -x_14 = l_Lean_Meta_instantiateMVarsIfMVarApp(x_2, x_9, x_10, x_11, x_12, x_13); -x_15 = lean_ctor_get(x_14, 0); -lean_inc(x_15); -x_16 = lean_ctor_get(x_14, 1); -lean_inc(x_16); -lean_dec(x_14); -x_17 = l_Lean_Expr_cleanupAnnotations(x_15); +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_13 = l_Lean_Meta_instantiateMVarsIfMVarApp(x_1, x_8, x_9, x_10, x_11, x_12); +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_13, 1); +lean_inc(x_15); +lean_dec(x_13); +x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_getNatOrBvValue_x3f___closed__1; +x_17 = l_Lean_Expr_cleanupAnnotations(x_14); x_18 = l_Lean_Expr_isApp(x_17); if (x_18 == 0) { lean_object* x_19; lean_object* x_20; lean_dec(x_17); -lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); +lean_dec(x_2); x_19 = lean_box(0); -x_20 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection___lambda__2(x_1, x_19, x_8, x_9, x_10, x_11, x_12, x_16); +x_20 = lean_apply_7(x_16, x_19, x_7, x_8, x_9, x_10, x_11, x_15); return x_20; } else @@ -8851,115 +8826,91 @@ lean_dec(x_21); if (x_23 == 0) { lean_object* x_24; lean_object* x_25; -lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); +lean_dec(x_2); x_24 = lean_box(0); -x_25 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection___lambda__2(x_1, x_24, x_8, x_9, x_10, x_11, x_12, x_16); +x_25 = lean_apply_7(x_16, x_24, x_7, x_8, x_9, x_10, x_11, x_15); return x_25; } else { lean_object* x_26; lean_object* x_27; -lean_dec(x_1); x_26 = lean_box(0); -x_27 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection___lambda__1(x_4, x_3, x_5, x_6, x_7, x_26, x_8, x_9, x_10, x_11, x_12, x_16); +x_27 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection___lambda__1(x_3, x_2, x_4, x_5, x_6, x_26, x_7, x_8, x_9, x_10, x_11, x_15); return x_27; } } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftConstReflection(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftConstReflection(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_14; -lean_inc(x_12); +lean_object* x_13; lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_getNatOrBvValue_x3f(x_2, x_3, x_8, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_14) == 0) +lean_inc(x_7); +x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_getNatOrBvValue_x3f(x_1, x_2, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_13) == 0) { -lean_object* x_15; -x_15 = lean_ctor_get(x_14, 0); -lean_inc(x_15); -if (lean_obj_tag(x_15) == 0) +lean_object* x_14; +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +if (lean_obj_tag(x_14) == 0) { -lean_object* x_16; lean_object* x_17; +uint8_t x_15; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_16 = lean_ctor_get(x_14, 1); -lean_inc(x_16); -lean_dec(x_14); -x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_8, x_9, x_10, x_11, x_12, x_16); -if (lean_obj_tag(x_17) == 0) -{ -uint8_t x_18; -x_18 = !lean_is_exclusive(x_17); -if (x_18 == 0) -{ -return x_17; -} -else -{ -lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_19 = lean_ctor_get(x_17, 0); -x_20 = lean_ctor_get(x_17, 1); -lean_inc(x_20); -lean_inc(x_19); -lean_dec(x_17); -x_21 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_21, 0, x_19); -lean_ctor_set(x_21, 1, x_20); -return x_21; -} -} -else -{ -uint8_t x_22; -x_22 = !lean_is_exclusive(x_17); -if (x_22 == 0) +lean_dec(x_3); +x_15 = !lean_is_exclusive(x_13); +if (x_15 == 0) { -return x_17; +lean_object* x_16; lean_object* x_17; +x_16 = lean_ctor_get(x_13, 0); +lean_dec(x_16); +x_17 = lean_box(0); +lean_ctor_set(x_13, 0, x_17); +return x_13; } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_17, 0); -x_24 = lean_ctor_get(x_17, 1); -lean_inc(x_24); -lean_inc(x_23); -lean_dec(x_17); -x_25 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_25, 0, x_23); -lean_ctor_set(x_25, 1, x_24); -return x_25; -} +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_13, 1); +lean_inc(x_18); +lean_dec(x_13); +x_19 = lean_box(0); +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_19); +lean_ctor_set(x_20, 1, x_18); +return x_20; } } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -lean_dec(x_1); -x_26 = lean_ctor_get(x_14, 1); -lean_inc(x_26); +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_13, 1); +lean_inc(x_21); +lean_dec(x_13); +x_22 = lean_ctor_get(x_14, 0); +lean_inc(x_22); lean_dec(x_14); -x_27 = lean_ctor_get(x_15, 0); -lean_inc(x_27); -lean_dec(x_15); -x_28 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftConstLikeReflection(x_27, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_26); -return x_28; +x_23 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftConstLikeReflection(x_22, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_21); +return x_23; } } else { -uint8_t x_29; -lean_dec(x_12); +uint8_t x_24; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -8968,24 +8919,24 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_1); -x_29 = !lean_is_exclusive(x_14); -if (x_29 == 0) +lean_dec(x_3); +x_24 = !lean_is_exclusive(x_13); +if (x_24 == 0) { -return x_14; +return x_13; } else { -lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_30 = lean_ctor_get(x_14, 0); -x_31 = lean_ctor_get(x_14, 1); -lean_inc(x_31); -lean_inc(x_30); -lean_dec(x_14); -x_32 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_32, 0, x_30); -lean_ctor_set(x_32, 1, x_31); -return x_32; +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_13, 0); +x_26 = lean_ctor_get(x_13, 1); +lean_inc(x_26); +lean_inc(x_25); +lean_dec(x_13); +x_27 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +return x_27; } } } @@ -8995,7 +8946,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_s { lean_object* x_12; lean_inc(x_2); -x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofOrAtom(x_2, x_6, x_7, x_8, x_9, x_10, x_11); +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(x_2, x_6, x_7, x_8, x_9, x_10, x_11); if (lean_obj_tag(x_12) == 0) { lean_object* x_13; @@ -9273,94 +9224,71 @@ return x_90; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_rotateReflection(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_rotateReflection(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_13; -lean_inc(x_11); +lean_object* x_12; lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -x_13 = l_Lean_Meta_getNatValue_x3f(x_2, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_13) == 0) +lean_inc(x_7); +x_12 = l_Lean_Meta_getNatValue_x3f(x_1, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_12) == 0) { -lean_object* x_14; -x_14 = lean_ctor_get(x_13, 0); -lean_inc(x_14); -if (lean_obj_tag(x_14) == 0) +lean_object* x_13; +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +if (lean_obj_tag(x_13) == 0) { -lean_object* x_15; lean_object* x_16; +uint8_t x_14; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_15 = lean_ctor_get(x_13, 1); -lean_inc(x_15); -lean_dec(x_13); -x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_7, x_8, x_9, x_10, x_11, x_15); -if (lean_obj_tag(x_16) == 0) -{ -uint8_t x_17; -x_17 = !lean_is_exclusive(x_16); -if (x_17 == 0) -{ -return x_16; -} -else -{ -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_16, 0); -x_19 = lean_ctor_get(x_16, 1); -lean_inc(x_19); -lean_inc(x_18); -lean_dec(x_16); -x_20 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_20, 0, x_18); -lean_ctor_set(x_20, 1, x_19); -return x_20; -} -} -else -{ -uint8_t x_21; -x_21 = !lean_is_exclusive(x_16); -if (x_21 == 0) +lean_dec(x_2); +x_14 = !lean_is_exclusive(x_12); +if (x_14 == 0) { -return x_16; +lean_object* x_15; lean_object* x_16; +x_15 = lean_ctor_get(x_12, 0); +lean_dec(x_15); +x_16 = lean_box(0); +lean_ctor_set(x_12, 0, x_16); +return x_12; } else { -lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_22 = lean_ctor_get(x_16, 0); -x_23 = lean_ctor_get(x_16, 1); -lean_inc(x_23); -lean_inc(x_22); -lean_dec(x_16); -x_24 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_24, 0, x_22); -lean_ctor_set(x_24, 1, x_23); -return x_24; -} +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_12, 1); +lean_inc(x_17); +lean_dec(x_12); +x_18 = lean_box(0); +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set(x_19, 1, x_17); +return x_19; } } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -lean_dec(x_1); -x_25 = lean_ctor_get(x_13, 1); -lean_inc(x_25); +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_12, 1); +lean_inc(x_20); +lean_dec(x_12); +x_21 = lean_ctor_get(x_13, 0); +lean_inc(x_21); lean_dec(x_13); -x_26 = lean_ctor_get(x_14, 0); -lean_inc(x_26); -lean_dec(x_14); -x_27 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftConstLikeReflection(x_26, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_25); -return x_27; +x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftConstLikeReflection(x_21, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_20); +return x_22; } } else { -uint8_t x_28; -lean_dec(x_11); +uint8_t x_23; lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -9369,78 +9297,69 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_1); -x_28 = !lean_is_exclusive(x_13); -if (x_28 == 0) +lean_dec(x_2); +x_23 = !lean_is_exclusive(x_12); +if (x_23 == 0) { -return x_13; +return x_12; } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_13, 0); -x_30 = lean_ctor_get(x_13, 1); -lean_inc(x_30); -lean_inc(x_29); -lean_dec(x_13); -x_31 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_31, 0, x_29); -lean_ctor_set(x_31, 1, x_30); -return x_31; -} -} +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_12, 0); +x_25 = lean_ctor_get(x_12, 1); +lean_inc(x_25); +lean_inc(x_24); +lean_dec(x_12); +x_26 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_26, 0, x_24); +lean_ctor_set(x_26, 1, x_25); +return x_26; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_3); -return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_10; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_3); -return x_10; +lean_object* x_9; +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_2); +return x_9; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_10; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_object* x_9; +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_2); -return x_10; +return x_9; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_10; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_3); -return x_10; +lean_object* x_9; +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_1); +return x_9; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__31___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; -x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__31(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_2); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__32___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__32___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; -x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__32(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__32(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_2); return x_9; } @@ -9464,22 +9383,21 @@ lean_dec(x_6); return x_13; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_rotateReflection___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_9; -x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_2); -return x_9; +lean_object* x_12; +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_rotateReflection(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_1); +return x_12; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_rotateReflection___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { -lean_object* x_13; -x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_rotateReflection(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_2); -return x_13; +lean_object* x_8; +x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +return x_8; } } lean_object* initialize_Lean_Elab_Tactic_BVDecide_Frontend_BVDecide_Reflect(uint8_t builtin, lean_object*); @@ -9551,264 +9469,292 @@ l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goBvLit___closed__5 = _ini lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goBvLit___closed__5); l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goBvLit___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goBvLit___closed__6(); lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goBvLit___closed__6); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__6); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__7); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__5___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__5___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__5___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__5___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__5___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__5___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__7___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__7___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__7___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__7___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__7___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__7___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__9___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__9___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__9___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__9___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__9___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__9___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__11___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__11___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__11___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__11___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__11___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__11___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__6); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__7); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__8(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__8); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__9 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__9(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__9); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__10 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__10(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__10); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__6); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__7); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__8(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__8); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__9 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__9(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__9); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__10 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__10(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__10); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__23___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__23___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__23___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__23___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__23___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__23___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__24___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__24___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__24___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__24___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__24___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__24___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__25___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__25___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__25___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__25___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__25___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__25___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__26___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__26___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__26___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__26___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__26___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__26___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__27___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__27___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__27___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__27___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__27___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__27___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__28___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__28___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__28___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__28___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__28___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__28___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__29___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__29___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__29___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__29___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__29___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__29___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__30___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__30___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__30___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__30___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__30___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__30___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__6); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__7); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__8(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__8); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__9 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__9(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__9); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__10 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__10(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__10); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__11 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__11(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__11); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__12 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__12(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__12); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__13 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__13(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__13); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__14 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__14(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__14); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__15 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__15(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__15); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__16 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__16(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__16); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__17 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__17(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__17); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__18 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__18(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__18); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__19 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__19(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__19); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__20 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__20(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__20); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__21 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__21(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__21); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__22 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__22(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__22); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__23 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__23(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__23); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__24 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__24(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__24); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__25 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__25(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__25); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__26 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__26(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__26); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__27 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__27(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__27); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__28 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__28(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__28); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__29 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__29(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__29); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__30 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__30(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__30); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__31 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__31(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__31); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__32 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__32(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__32); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__33 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__33(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__33); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__34 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__34(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__34); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__35 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__35(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__35); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__36 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__36(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__36); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__37 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__37(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__37); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__38 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__38(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__38); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__39 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__39(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__39); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__40 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__40(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__40); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__41 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__41(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__41); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__42 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__42(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__42); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__43 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__43(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__43); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__44 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__44(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__44); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__45 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__45(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__45); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__46 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__46(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__46); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__47 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__47(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__47); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__48 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__48(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__48); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__49 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__49(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__49); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__50 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__50(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__50); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__51 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__51(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__51); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__7); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__5___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__5___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__5___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__5___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__5___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__5___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__7___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__7___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__7___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__7___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__7___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__7___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__9___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__9___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__9___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__9___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__9___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__9___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__7); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__8(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__8); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__9 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__9(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__9); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__10 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__10(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__10); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__7); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__8(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__8); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__9 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__9(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__9); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__10 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__10(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__10); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__23___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__23___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__23___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__23___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__23___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__23___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__24___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__24___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__24___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__24___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__24___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__24___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__25___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__25___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__25___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__25___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__25___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__25___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__26___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__26___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__26___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__26___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__26___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__26___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__27___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__27___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__27___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__27___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__27___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__27___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__28___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__28___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__28___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__28___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__28___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__28___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__29___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__29___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__29___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__29___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__29___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__29___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__30___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__30___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__30___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__30___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__30___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__30___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__31___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__31___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__31___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__31___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__31___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__31___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__7); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__8(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__8); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__9 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__9(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__9); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__10 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__10(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__10); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__11 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__11(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__11); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__12 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__12(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__12); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__13 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__13(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__13); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__14 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__14(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__14); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__15 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__15(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__15); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__16 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__16(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__16); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__17 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__17(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__17); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__18 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__18(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__18); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__19 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__19(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__19); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__20 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__20(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__20); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__21 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__21(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__21); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__22 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__22(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__22); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__23 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__23(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__23); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__24 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__24(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__24); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__25 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__25(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__25); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__26 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__26(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__26); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__27 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__27(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__27); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__28 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__28(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__28); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__29 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__29(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__29); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__30 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__30(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__30); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__31 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__31(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__31); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__32 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__32(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__32); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__33 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__33(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__33); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__34 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__34(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__34); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__35 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__35(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__35); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__36 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__36(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__36); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__37 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__37(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__37); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__38 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__38(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__38); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__39 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__39(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__39); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__40 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__40(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__40); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__41 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__41(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__41); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__42 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__42(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__42); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__43 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__43(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__43); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__44 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__44(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__44); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__45 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__45(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__45); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__46 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__46(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__46); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__47 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__47(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__47); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__48 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__48(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__48); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__49 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__49(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__49); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__50 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__50(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__50); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__51 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__51(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__51); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__52 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__52(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__52); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__53 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__53(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__53); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__54 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__54(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__54); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__55 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__55(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__55); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__56 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__56(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__56); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__57 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__57(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__57); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__58 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__58(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__58); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__59 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__59(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__59); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__60 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__60(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__60); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__61 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__61(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__61); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__62 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__62(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__62); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__63 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__63(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__63); l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__1(); lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__1); l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__2(); @@ -9859,6 +9805,10 @@ l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed_ lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__24); l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__25 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__25(); lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__25); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__26 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__26(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__26); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__27 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__27(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__27); l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_unaryReflection___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_unaryReflection___closed__1(); lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_unaryReflection___closed__1); l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_unaryReflection___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_unaryReflection___closed__2(); diff --git a/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/ReifiedBVLogical.c b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/ReifiedBVLogical.c index 14b9500fffe9..aeaede831620 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/ReifiedBVLogical.c +++ b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/ReifiedBVLogical.c @@ -13,132 +13,138 @@ #ifdef __cplusplus extern "C" { #endif +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__8; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__6; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goOrAtom(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__5; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__4; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__6; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__9; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__9; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkTrans(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__3; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__12; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__2; lean_object* l_Lean_mkAppB(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__11; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4___closed__1; uint8_t l_Lean_Expr_isApp(lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__7___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__8; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__5___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4___closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__5___closed__2; +lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__4; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__4; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__5; +LEAN_EXPORT lean_object* l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_cleanupAnnotations(lean_object*); lean_object* l_Lean_mkApp4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__5; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__1; -LEAN_EXPORT lean_object* l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__11; lean_object* l_Lean_Level_ofNat(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__9; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__6; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__5; lean_object* l_Lean_mkApp6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__6; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkTrans___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__9; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkTrans___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__6___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__2; lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_M_atomsAssignment(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__12; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl(lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; lean_object* l_Lean_Expr_appArg(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__1; lean_object* l_Lean_Expr_appFnCleanup(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__9; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__4; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__2; +LEAN_EXPORT lean_object* l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___spec__1(lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__10; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__7; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__5; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__2; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__10; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__1; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__6; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_boolAtom(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__7___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4___closed__2; -LEAN_EXPORT lean_object* l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__8; lean_object* l_Lean_mkApp3(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__8; lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__6; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__7; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__6___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4___closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__8; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isConstOf(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__1; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__3; -LEAN_EXPORT lean_object* l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___spec__1(lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__6; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__7___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__5; lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__7; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__1; lean_object* l_Lean_Meta_instantiateMVarsIfMVarApp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__7; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__5; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__13; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__7___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__6; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__7; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__8; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__6___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__6; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__5; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__13; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__5; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkTrans___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__6; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__6; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__3; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__10; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__4; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__1; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__4; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__9; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__5___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__5; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__6___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__7; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__5___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__4; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__3; static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__1() { _start: { @@ -380,7 +386,7 @@ lean_dec(x_2); return x_8; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__1() { _start: { lean_object* x_1; @@ -388,7 +394,7 @@ x_1 = lean_mk_string_unchecked("BoolExpr", 8, 8); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__2() { _start: { lean_object* x_1; @@ -396,30 +402,30 @@ x_1 = lean_mk_string_unchecked("literal", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__2; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__2; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__3; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__3; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__5() { _start: { lean_object* x_1; @@ -427,33 +433,103 @@ x_1 = lean_mk_string_unchecked("BVPred", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__6() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__5; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__5; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__6; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__6; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_1); +if (x_8 == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_9 = lean_ctor_get(x_1, 0); +x_10 = lean_ctor_get(x_1, 2); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_9); +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__4; +x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7; +x_14 = l_Lean_mkAppB(x_12, x_13, x_10); +lean_ctor_set(x_1, 2, x_14); +lean_ctor_set(x_1, 0, x_11); +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_1); +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_16, 1, x_7); +return x_16; +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_17 = lean_ctor_get(x_1, 0); +x_18 = lean_ctor_get(x_1, 1); +x_19 = lean_ctor_get(x_1, 2); +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_dec(x_1); +x_20 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_20, 0, x_17); +x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__4; +x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7; +x_23 = l_Lean_mkAppB(x_21, x_22, x_19); +x_24 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_24, 0, x_20); +lean_ctor_set(x_24, 1, x_18); +lean_ctor_set(x_24, 2, x_23); +x_25 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_25, 0, x_24); +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_7); +return x_26; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; -x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_boolAtom(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom(x_1, x_2, x_3, x_4, x_5, x_6, x_7); if (lean_obj_tag(x_8) == 0) { lean_object* x_9; @@ -462,6 +538,11 @@ lean_inc(x_9); if (lean_obj_tag(x_9) == 0) { uint8_t x_10; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); x_10 = !lean_is_exclusive(x_8); if (x_10 == 0) { @@ -487,1235 +568,1221 @@ return x_15; } else { -uint8_t x_16; -x_16 = !lean_is_exclusive(x_9); -if (x_16 == 0) -{ -uint8_t x_17; -x_17 = !lean_is_exclusive(x_8); -if (x_17 == 0) -{ -lean_object* x_18; lean_object* x_19; uint8_t x_20; -x_18 = lean_ctor_get(x_9, 0); -x_19 = lean_ctor_get(x_8, 0); -lean_dec(x_19); -x_20 = !lean_is_exclusive(x_18); -if (x_20 == 0) -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_21 = lean_ctor_get(x_18, 0); -x_22 = lean_ctor_get(x_18, 2); -x_23 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_23, 0, x_21); -x_24 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__4; -x_25 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -x_26 = l_Lean_mkAppB(x_24, x_25, x_22); -lean_ctor_set(x_18, 2, x_26); -lean_ctor_set(x_18, 0, x_23); -return x_8; -} -else -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_27 = lean_ctor_get(x_18, 0); -x_28 = lean_ctor_get(x_18, 1); -x_29 = lean_ctor_get(x_18, 2); -lean_inc(x_29); -lean_inc(x_28); -lean_inc(x_27); -lean_dec(x_18); -x_30 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_30, 0, x_27); -x_31 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__4; -x_32 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -x_33 = l_Lean_mkAppB(x_31, x_32, x_29); -x_34 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_34, 0, x_30); -lean_ctor_set(x_34, 1, x_28); -lean_ctor_set(x_34, 2, x_33); -lean_ctor_set(x_9, 0, x_34); -return x_8; -} -} -else -{ -lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_35 = lean_ctor_get(x_9, 0); -x_36 = lean_ctor_get(x_8, 1); -lean_inc(x_36); +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_8, 1); +lean_inc(x_16); lean_dec(x_8); -x_37 = lean_ctor_get(x_35, 0); -lean_inc(x_37); -x_38 = lean_ctor_get(x_35, 1); -lean_inc(x_38); -x_39 = lean_ctor_get(x_35, 2); -lean_inc(x_39); -if (lean_is_exclusive(x_35)) { - lean_ctor_release(x_35, 0); - lean_ctor_release(x_35, 1); - lean_ctor_release(x_35, 2); - x_40 = x_35; -} else { - lean_dec_ref(x_35); - x_40 = lean_box(0); -} -x_41 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_41, 0, x_37); -x_42 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__4; -x_43 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -x_44 = l_Lean_mkAppB(x_42, x_43, x_39); -if (lean_is_scalar(x_40)) { - x_45 = lean_alloc_ctor(0, 3, 0); -} else { - x_45 = x_40; -} -lean_ctor_set(x_45, 0, x_41); -lean_ctor_set(x_45, 1, x_38); -lean_ctor_set(x_45, 2, x_44); -lean_ctor_set(x_9, 0, x_45); -x_46 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_46, 0, x_9); -lean_ctor_set(x_46, 1, x_36); -return x_46; -} -} -else -{ -lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_47 = lean_ctor_get(x_9, 0); -lean_inc(x_47); +x_17 = lean_ctor_get(x_9, 0); +lean_inc(x_17); lean_dec(x_9); -x_48 = lean_ctor_get(x_8, 1); -lean_inc(x_48); -if (lean_is_exclusive(x_8)) { - lean_ctor_release(x_8, 0); - lean_ctor_release(x_8, 1); - x_49 = x_8; -} else { - lean_dec_ref(x_8); - x_49 = lean_box(0); -} -x_50 = lean_ctor_get(x_47, 0); -lean_inc(x_50); -x_51 = lean_ctor_get(x_47, 1); -lean_inc(x_51); -x_52 = lean_ctor_get(x_47, 2); -lean_inc(x_52); -if (lean_is_exclusive(x_47)) { - lean_ctor_release(x_47, 0); - lean_ctor_release(x_47, 1); - lean_ctor_release(x_47, 2); - x_53 = x_47; -} else { - lean_dec_ref(x_47); - x_53 = lean_box(0); -} -x_54 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_54, 0, x_50); -x_55 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__4; -x_56 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -x_57 = l_Lean_mkAppB(x_55, x_56, x_52); -if (lean_is_scalar(x_53)) { - x_58 = lean_alloc_ctor(0, 3, 0); -} else { - x_58 = x_53; -} -lean_ctor_set(x_58, 0, x_54); -lean_ctor_set(x_58, 1, x_51); -lean_ctor_set(x_58, 2, x_57); -x_59 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_59, 0, x_58); -if (lean_is_scalar(x_49)) { - x_60 = lean_alloc_ctor(0, 2, 0); -} else { - x_60 = x_49; -} -lean_ctor_set(x_60, 0, x_59); -lean_ctor_set(x_60, 1, x_48); -return x_60; -} +x_18 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred(x_17, x_2, x_3, x_4, x_5, x_6, x_16); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_18; } } else { -uint8_t x_61; -x_61 = !lean_is_exclusive(x_8); -if (x_61 == 0) +uint8_t x_19; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_19 = !lean_is_exclusive(x_8); +if (x_19 == 0) { return x_8; } else { -lean_object* x_62; lean_object* x_63; lean_object* x_64; -x_62 = lean_ctor_get(x_8, 0); -x_63 = lean_ctor_get(x_8, 1); -lean_inc(x_63); -lean_inc(x_62); +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_8, 0); +x_21 = lean_ctor_get(x_8, 1); +lean_inc(x_21); +lean_inc(x_20); lean_dec(x_8); -x_64 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_64, 0, x_62); -lean_ctor_set(x_64, 1, x_63); -return x_64; +x_22 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_22, 0, x_20); +lean_ctor_set(x_22, 1, x_21); +return x_22; } } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr(x_1, x_9, x_10, x_11, x_12, x_13, x_14); -x_16 = lean_ctor_get(x_15, 0); -lean_inc(x_16); -x_17 = lean_ctor_get(x_15, 1); -lean_inc(x_17); -lean_dec(x_15); -x_18 = lean_ctor_get(x_2, 1); -lean_inc(x_18); -lean_dec(x_2); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); +lean_object* x_8; +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +if (lean_obj_tag(x_8) == 0) +{ +lean_object* x_9; +x_9 = lean_ctor_get(x_8, 0); lean_inc(x_9); -x_19 = lean_apply_6(x_18, x_9, x_10, x_11, x_12, x_13, x_17); -if (lean_obj_tag(x_19) == 0) +if (lean_obj_tag(x_9) == 0) { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_19, 1); -lean_inc(x_21); -lean_dec(x_19); -x_22 = lean_ctor_get(x_3, 1); -lean_inc(x_22); +uint8_t x_10; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); -x_23 = lean_apply_6(x_22, x_9, x_10, x_11, x_12, x_13, x_21); -if (lean_obj_tag(x_23) == 0) -{ -uint8_t x_24; -x_24 = !lean_is_exclusive(x_23); -if (x_24 == 0) +lean_dec(x_2); +x_10 = !lean_is_exclusive(x_8); +if (x_10 == 0) { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_23, 0); -x_26 = l_Lean_Expr_const___override(x_4, x_5); -x_27 = l_Lean_mkApp6(x_26, x_6, x_7, x_8, x_16, x_20, x_25); -lean_ctor_set(x_23, 0, x_27); -return x_23; +lean_object* x_11; lean_object* x_12; +x_11 = lean_ctor_get(x_8, 0); +lean_dec(x_11); +x_12 = lean_box(0); +lean_ctor_set(x_8, 0, x_12); +return x_8; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_28 = lean_ctor_get(x_23, 0); -x_29 = lean_ctor_get(x_23, 1); -lean_inc(x_29); -lean_inc(x_28); -lean_dec(x_23); -x_30 = l_Lean_Expr_const___override(x_4, x_5); -x_31 = l_Lean_mkApp6(x_30, x_6, x_7, x_8, x_16, x_20, x_28); -x_32 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_32, 0, x_31); -lean_ctor_set(x_32, 1, x_29); -return x_32; +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_8, 1); +lean_inc(x_13); +lean_dec(x_8); +x_14 = lean_box(0); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_13); +return x_15; } } else { -uint8_t x_33; -lean_dec(x_20); -lean_dec(x_16); +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_8, 1); +lean_inc(x_16); lean_dec(x_8); -lean_dec(x_7); +x_17 = lean_ctor_get(x_9, 0); +lean_inc(x_17); +lean_dec(x_9); +x_18 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred(x_17, x_2, x_3, x_4, x_5, x_6, x_16); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_33 = !lean_is_exclusive(x_23); -if (x_33 == 0) -{ -return x_23; -} -else -{ -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_23, 0); -x_35 = lean_ctor_get(x_23, 1); -lean_inc(x_35); -lean_inc(x_34); -lean_dec(x_23); -x_36 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_36, 0, x_34); -lean_ctor_set(x_36, 1, x_35); -return x_36; -} +lean_dec(x_3); +lean_dec(x_2); +return x_18; } } else { -uint8_t x_37; -lean_dec(x_16); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); +uint8_t x_19; lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_37 = !lean_is_exclusive(x_19); -if (x_37 == 0) +lean_dec(x_2); +x_19 = !lean_is_exclusive(x_8); +if (x_19 == 0) { -return x_19; +return x_8; } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_19, 0); -x_39 = lean_ctor_get(x_19, 1); -lean_inc(x_39); -lean_inc(x_38); -lean_dec(x_19); -x_40 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_40, 0, x_38); -lean_ctor_set(x_40, 1, x_39); -return x_40; +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_8, 0); +x_21 = lean_ctor_get(x_8, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_8); +x_22 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_22, 0, x_20); +lean_ctor_set(x_22, 1, x_21); +return x_22; } } } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__1() { +LEAN_EXPORT lean_object* l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("gate", 4, 4); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__2() { +lean_object* x_8; +x_8 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_8, 0, x_1); +lean_ctor_set(x_8, 1, x_7); +return x_8; +} +} +LEAN_EXPORT lean_object* l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___spec__1(lean_object* x_1) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__1; -x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); -return x_6; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___spec__1___rarg___boxed), 7, 0); +return x_2; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3() { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__2; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; +lean_object* x_9; +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred(x_1, x_3, x_4, x_5, x_6, x_7, x_8); +return x_9; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("Gate", 4, 4); +x_1 = lean_mk_string_unchecked("Reflect", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__2() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("and", 3, 3); +x_1 = lean_mk_string_unchecked("beq_congr", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__6() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__3() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__4; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__5; -x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); -return x_6; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__2; +x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); +return x_7; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__7() { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +uint8_t x_10; lean_object* x_11; lean_object* x_12; +x_10 = 2; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__3; +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection(x_1, x_2, x_10, x_11, x_4, x_5, x_6, x_7, x_8, x_9); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; lean_object* x_9; +x_8 = lean_box(0); +x_9 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_9, 0, x_8); +lean_ctor_set(x_9, 1, x_7); +return x_9; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__3___boxed), 7, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("BitVec", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__6; -x_3 = l_Lean_Expr_const___override(x_2, x_1); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4___closed__2; +x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__8() { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_11 = l_Lean_Meta_instantiateMVarsIfMVarApp(x_2, x_6, x_7, x_8, x_9, x_10); +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4___closed__1; +x_15 = l_Lean_Expr_cleanupAnnotations(x_12); +x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__8; +x_17 = l_Lean_Expr_isConstOf(x_15, x_16); +if (x_17 == 0) +{ +uint8_t x_18; +lean_dec(x_4); +lean_dec(x_3); +x_18 = l_Lean_Expr_isApp(x_15); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; +lean_dec(x_15); +lean_dec(x_1); +x_19 = lean_box(0); +x_20 = lean_apply_7(x_14, x_19, x_5, x_6, x_7, x_8, x_9, x_13); +return x_20; +} +else +{ +lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_21 = l_Lean_Expr_appFnCleanup(x_15, lean_box(0)); +x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4___closed__3; +x_23 = l_Lean_Expr_isConstOf(x_21, x_22); +lean_dec(x_21); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; +lean_dec(x_1); +x_24 = lean_box(0); +x_25 = lean_apply_7(x_14, x_24, x_5, x_6, x_7, x_8, x_9, x_13); +return x_25; +} +else +{ +lean_object* x_26; +x_26 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred(x_1, x_5, x_6, x_7, x_8, x_9, x_13); +return x_26; +} +} +} +else +{ +lean_object* x_27; lean_object* x_28; +lean_dec(x_15); +lean_dec(x_1); +x_27 = lean_box(0); +x_28 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2(x_3, x_4, x_27, x_5, x_6, x_7, x_8, x_9, x_13); +return x_28; +} +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__5___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("xor", 3, 3); +x_1 = lean_mk_string_unchecked("xor_congr", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__9() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__5___closed__2() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__4; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__8; -x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); -return x_6; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__5___closed__1; +x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); +return x_7; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__10() { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__9; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; +uint8_t x_9; lean_object* x_10; lean_object* x_11; +x_9 = 1; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__5___closed__2; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection(x_1, x_2, x_9, x_10, x_3, x_4, x_5, x_6, x_7, x_8); +return x_11; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__11() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__6___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("beq", 3, 3); +x_1 = lean_mk_string_unchecked("and_congr", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__12() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__6___closed__2() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__4; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__11; -x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); -return x_6; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__6___closed__1; +x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); +return x_7; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__13() { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__12; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; +uint8_t x_9; lean_object* x_10; lean_object* x_11; +x_9 = 0; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__6___closed__2; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection(x_1, x_2, x_9, x_10, x_3, x_4, x_5, x_6, x_7, x_8); +return x_11; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__7___closed__1() { _start: { -lean_object* x_11; -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_1); -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of(x_1, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_11) == 0) +lean_object* x_1; +x_1 = lean_mk_string_unchecked("not_congr", 9, 9); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__7___closed__2() { +_start: { -lean_object* x_12; -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__7___closed__1; +x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; +x_11 = lean_ctor_get(x_1, 1); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_apply_6(x_11, x_5, x_6, x_7, x_8, x_9, x_10); if (lean_obj_tag(x_12) == 0) { uint8_t x_13; -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -x_13 = !lean_is_exclusive(x_11); +x_13 = !lean_is_exclusive(x_12); if (x_13 == 0) { -lean_object* x_14; lean_object* x_15; -x_14 = lean_ctor_get(x_11, 0); -lean_dec(x_14); -x_15 = lean_box(0); -lean_ctor_set(x_11, 0, x_15); -return x_11; +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_14 = lean_ctor_get(x_12, 0); +x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__7___closed__2; +x_16 = l_Lean_Expr_const___override(x_15, x_2); +x_17 = l_Lean_mkApp3(x_16, x_3, x_4, x_14); +lean_ctor_set(x_12, 0, x_17); +return x_12; } else { -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_11, 1); -lean_inc(x_16); -lean_dec(x_11); -x_17 = lean_box(0); -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_17); -lean_ctor_set(x_18, 1, x_16); -return x_18; +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_18 = lean_ctor_get(x_12, 0); +x_19 = lean_ctor_get(x_12, 1); +lean_inc(x_19); +lean_inc(x_18); +lean_dec(x_12); +x_20 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__7___closed__2; +x_21 = l_Lean_Expr_const___override(x_20, x_2); +x_22 = l_Lean_mkApp3(x_21, x_3, x_4, x_18); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_19); +return x_23; } } else { -lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_19 = lean_ctor_get(x_11, 1); -lean_inc(x_19); -lean_dec(x_11); -x_20 = lean_ctor_get(x_12, 0); -lean_inc(x_20); -lean_dec(x_12); -lean_inc(x_2); -x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of(x_2, x_5, x_6, x_7, x_8, x_9, x_19); -if (lean_obj_tag(x_21) == 0) -{ -lean_object* x_22; -x_22 = lean_ctor_get(x_21, 0); -lean_inc(x_22); -if (lean_obj_tag(x_22) == 0) -{ -uint8_t x_23; -lean_dec(x_20); +uint8_t x_24; lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_23 = !lean_is_exclusive(x_21); -if (x_23 == 0) +x_24 = !lean_is_exclusive(x_12); +if (x_24 == 0) { -lean_object* x_24; lean_object* x_25; -x_24 = lean_ctor_get(x_21, 0); -lean_dec(x_24); -x_25 = lean_box(0); -lean_ctor_set(x_21, 0, x_25); -return x_21; +return x_12; } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_21, 1); +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_12, 0); +x_26 = lean_ctor_get(x_12, 1); lean_inc(x_26); -lean_dec(x_21); -x_27 = lean_box(0); -x_28 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_28, 0, x_27); -lean_ctor_set(x_28, 1, x_26); -return x_28; +lean_inc(x_25); +lean_dec(x_12); +x_27 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +return x_27; } } -else -{ -uint8_t x_29; -x_29 = !lean_is_exclusive(x_21); -if (x_29 == 0) -{ -lean_object* x_30; uint8_t x_31; -x_30 = lean_ctor_get(x_21, 0); -lean_dec(x_30); -x_31 = !lean_is_exclusive(x_22); -if (x_31 == 0) +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__1() { +_start: { -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_32 = lean_ctor_get(x_22, 0); -x_33 = lean_ctor_get(x_20, 0); -lean_inc(x_33); -x_34 = lean_ctor_get(x_32, 0); -lean_inc(x_34); -x_35 = lean_alloc_ctor(3, 2, 1); -lean_ctor_set(x_35, 0, x_33); -lean_ctor_set(x_35, 1, x_34); -lean_ctor_set_uint8(x_35, sizeof(void*)*2, x_3); -x_36 = lean_box(0); -x_37 = lean_ctor_get(x_20, 2); -lean_inc(x_37); -x_38 = lean_ctor_get(x_32, 2); -lean_inc(x_38); -lean_inc(x_37); -x_39 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___boxed), 7, 1); -lean_closure_set(x_39, 0, x_37); -lean_inc(x_38); -x_40 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___lambda__1), 14, 7); -lean_closure_set(x_40, 0, x_38); -lean_closure_set(x_40, 1, x_20); -lean_closure_set(x_40, 2, x_32); -lean_closure_set(x_40, 3, x_4); -lean_closure_set(x_40, 4, x_36); -lean_closure_set(x_40, 5, x_1); -lean_closure_set(x_40, 6, x_2); -x_41 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_41, 0, x_39); -lean_closure_set(x_41, 1, x_40); -switch (x_3) { -case 0: +lean_object* x_1; +x_1 = lean_mk_string_unchecked("not", 3, 3); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__2() { +_start: { -lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_42 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; -x_43 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -x_44 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__7; -x_45 = l_Lean_mkApp4(x_42, x_43, x_44, x_37, x_38); -x_46 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_46, 0, x_35); -lean_ctor_set(x_46, 1, x_41); -lean_ctor_set(x_46, 2, x_45); -lean_ctor_set(x_22, 0, x_46); -return x_21; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__1; +x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); +return x_6; } -case 1: +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__3() { +_start: { -lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_47 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; -x_48 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -x_49 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__10; -x_50 = l_Lean_mkApp4(x_47, x_48, x_49, x_37, x_38); -x_51 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_51, 0, x_35); -lean_ctor_set(x_51, 1, x_41); -lean_ctor_set(x_51, 2, x_50); -lean_ctor_set(x_22, 0, x_51); -return x_21; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__2; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; } -default: +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: { -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; -x_52 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; -x_53 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -x_54 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__13; -x_55 = l_Lean_mkApp4(x_52, x_53, x_54, x_37, x_38); -x_56 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_56, 0, x_35); -lean_ctor_set(x_56, 1, x_41); -lean_ctor_set(x_56, 2, x_55); -lean_ctor_set(x_22, 0, x_56); -return x_21; +lean_object* x_8; +lean_inc(x_1); +x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goOrAtom(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +if (lean_obj_tag(x_8) == 0) +{ +lean_object* x_9; +x_9 = lean_ctor_get(x_8, 0); +lean_inc(x_9); +if (lean_obj_tag(x_9) == 0) +{ +uint8_t x_10; +lean_dec(x_1); +x_10 = !lean_is_exclusive(x_8); +if (x_10 == 0) +{ +lean_object* x_11; lean_object* x_12; +x_11 = lean_ctor_get(x_8, 0); +lean_dec(x_11); +x_12 = lean_box(0); +lean_ctor_set(x_8, 0, x_12); +return x_8; } +else +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_8, 1); +lean_inc(x_13); +lean_dec(x_8); +x_14 = lean_box(0); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_13); +return x_15; } } else { -lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_57 = lean_ctor_get(x_22, 0); -lean_inc(x_57); -lean_dec(x_22); -x_58 = lean_ctor_get(x_20, 0); -lean_inc(x_58); -x_59 = lean_ctor_get(x_57, 0); -lean_inc(x_59); -x_60 = lean_alloc_ctor(3, 2, 1); -lean_ctor_set(x_60, 0, x_58); -lean_ctor_set(x_60, 1, x_59); -lean_ctor_set_uint8(x_60, sizeof(void*)*2, x_3); -x_61 = lean_box(0); -x_62 = lean_ctor_get(x_20, 2); -lean_inc(x_62); -x_63 = lean_ctor_get(x_57, 2); -lean_inc(x_63); -lean_inc(x_62); -x_64 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___boxed), 7, 1); -lean_closure_set(x_64, 0, x_62); -lean_inc(x_63); -x_65 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___lambda__1), 14, 7); -lean_closure_set(x_65, 0, x_63); -lean_closure_set(x_65, 1, x_20); -lean_closure_set(x_65, 2, x_57); -lean_closure_set(x_65, 3, x_4); -lean_closure_set(x_65, 4, x_61); -lean_closure_set(x_65, 5, x_1); -lean_closure_set(x_65, 6, x_2); -x_66 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_66, 0, x_64); -lean_closure_set(x_66, 1, x_65); -switch (x_3) { -case 0: +uint8_t x_16; +x_16 = !lean_is_exclusive(x_9); +if (x_16 == 0) { -lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; -x_67 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; -x_68 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -x_69 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__7; -x_70 = l_Lean_mkApp4(x_67, x_68, x_69, x_62, x_63); -x_71 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_71, 0, x_60); -lean_ctor_set(x_71, 1, x_66); -lean_ctor_set(x_71, 2, x_70); -x_72 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_72, 0, x_71); -lean_ctor_set(x_21, 0, x_72); -return x_21; -} -case 1: +uint8_t x_17; +x_17 = !lean_is_exclusive(x_8); +if (x_17 == 0) { -lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; -x_73 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; -x_74 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -x_75 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__10; -x_76 = l_Lean_mkApp4(x_73, x_74, x_75, x_62, x_63); -x_77 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_77, 0, x_60); -lean_ctor_set(x_77, 1, x_66); -lean_ctor_set(x_77, 2, x_76); -x_78 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_78, 0, x_77); -lean_ctor_set(x_21, 0, x_78); -return x_21; -} -default: +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; +x_18 = lean_ctor_get(x_9, 0); +x_19 = lean_ctor_get(x_8, 0); +lean_dec(x_19); +x_20 = lean_ctor_get(x_18, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_18, 2); +lean_inc(x_21); +x_22 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_22, 0, x_20); +x_23 = lean_box(0); +x_24 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__3; +x_25 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7; +lean_inc(x_21); +x_26 = l_Lean_mkAppB(x_24, x_25, x_21); +x_27 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___boxed), 7, 1); +lean_closure_set(x_27, 0, x_21); +lean_inc(x_18); +x_28 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__7), 10, 3); +lean_closure_set(x_28, 0, x_18); +lean_closure_set(x_28, 1, x_23); +lean_closure_set(x_28, 2, x_1); +x_29 = !lean_is_exclusive(x_18); +if (x_29 == 0) { -lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; -x_79 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; -x_80 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -x_81 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__13; -x_82 = l_Lean_mkApp4(x_79, x_80, x_81, x_62, x_63); -x_83 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_83, 0, x_60); -lean_ctor_set(x_83, 1, x_66); -lean_ctor_set(x_83, 2, x_82); -x_84 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_84, 0, x_83); -lean_ctor_set(x_21, 0, x_84); -return x_21; -} +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_30 = lean_ctor_get(x_18, 2); +lean_dec(x_30); +x_31 = lean_ctor_get(x_18, 1); +lean_dec(x_31); +x_32 = lean_ctor_get(x_18, 0); +lean_dec(x_32); +x_33 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_33, 0, x_27); +lean_closure_set(x_33, 1, x_28); +lean_ctor_set(x_18, 2, x_26); +lean_ctor_set(x_18, 1, x_33); +lean_ctor_set(x_18, 0, x_22); +return x_8; } +else +{ +lean_object* x_34; lean_object* x_35; +lean_dec(x_18); +x_34 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_34, 0, x_27); +lean_closure_set(x_34, 1, x_28); +x_35 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_35, 0, x_22); +lean_ctor_set(x_35, 1, x_34); +lean_ctor_set(x_35, 2, x_26); +lean_ctor_set(x_9, 0, x_35); +return x_8; } } else { -lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; -x_85 = lean_ctor_get(x_21, 1); -lean_inc(x_85); -lean_dec(x_21); -x_86 = lean_ctor_get(x_22, 0); -lean_inc(x_86); -if (lean_is_exclusive(x_22)) { - lean_ctor_release(x_22, 0); - x_87 = x_22; +lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_36 = lean_ctor_get(x_9, 0); +x_37 = lean_ctor_get(x_8, 1); +lean_inc(x_37); +lean_dec(x_8); +x_38 = lean_ctor_get(x_36, 0); +lean_inc(x_38); +x_39 = lean_ctor_get(x_36, 2); +lean_inc(x_39); +x_40 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_40, 0, x_38); +x_41 = lean_box(0); +x_42 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__3; +x_43 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7; +lean_inc(x_39); +x_44 = l_Lean_mkAppB(x_42, x_43, x_39); +x_45 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___boxed), 7, 1); +lean_closure_set(x_45, 0, x_39); +lean_inc(x_36); +x_46 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__7), 10, 3); +lean_closure_set(x_46, 0, x_36); +lean_closure_set(x_46, 1, x_41); +lean_closure_set(x_46, 2, x_1); +if (lean_is_exclusive(x_36)) { + lean_ctor_release(x_36, 0); + lean_ctor_release(x_36, 1); + lean_ctor_release(x_36, 2); + x_47 = x_36; } else { - lean_dec_ref(x_22); - x_87 = lean_box(0); + lean_dec_ref(x_36); + x_47 = lean_box(0); } -x_88 = lean_ctor_get(x_20, 0); -lean_inc(x_88); -x_89 = lean_ctor_get(x_86, 0); -lean_inc(x_89); -x_90 = lean_alloc_ctor(3, 2, 1); -lean_ctor_set(x_90, 0, x_88); -lean_ctor_set(x_90, 1, x_89); -lean_ctor_set_uint8(x_90, sizeof(void*)*2, x_3); -x_91 = lean_box(0); -x_92 = lean_ctor_get(x_20, 2); -lean_inc(x_92); -x_93 = lean_ctor_get(x_86, 2); -lean_inc(x_93); -lean_inc(x_92); -x_94 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___boxed), 7, 1); -lean_closure_set(x_94, 0, x_92); -lean_inc(x_93); -x_95 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___lambda__1), 14, 7); -lean_closure_set(x_95, 0, x_93); -lean_closure_set(x_95, 1, x_20); -lean_closure_set(x_95, 2, x_86); -lean_closure_set(x_95, 3, x_4); -lean_closure_set(x_95, 4, x_91); -lean_closure_set(x_95, 5, x_1); -lean_closure_set(x_95, 6, x_2); -x_96 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_96, 0, x_94); -lean_closure_set(x_96, 1, x_95); -switch (x_3) { -case 0: -{ -lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; -x_97 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; -x_98 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -x_99 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__7; -x_100 = l_Lean_mkApp4(x_97, x_98, x_99, x_92, x_93); -x_101 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_101, 0, x_90); -lean_ctor_set(x_101, 1, x_96); -lean_ctor_set(x_101, 2, x_100); -if (lean_is_scalar(x_87)) { - x_102 = lean_alloc_ctor(1, 1, 0); +x_48 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_48, 0, x_45); +lean_closure_set(x_48, 1, x_46); +if (lean_is_scalar(x_47)) { + x_49 = lean_alloc_ctor(0, 3, 0); } else { - x_102 = x_87; + x_49 = x_47; } -lean_ctor_set(x_102, 0, x_101); -x_103 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_103, 0, x_102); -lean_ctor_set(x_103, 1, x_85); -return x_103; +lean_ctor_set(x_49, 0, x_40); +lean_ctor_set(x_49, 1, x_48); +lean_ctor_set(x_49, 2, x_44); +lean_ctor_set(x_9, 0, x_49); +x_50 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_50, 0, x_9); +lean_ctor_set(x_50, 1, x_37); +return x_50; } -case 1: +} +else { -lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; -x_104 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; -x_105 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -x_106 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__10; -x_107 = l_Lean_mkApp4(x_104, x_105, x_106, x_92, x_93); -x_108 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_108, 0, x_90); -lean_ctor_set(x_108, 1, x_96); -lean_ctor_set(x_108, 2, x_107); -if (lean_is_scalar(x_87)) { - x_109 = lean_alloc_ctor(1, 1, 0); +lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; +x_51 = lean_ctor_get(x_9, 0); +lean_inc(x_51); +lean_dec(x_9); +x_52 = lean_ctor_get(x_8, 1); +lean_inc(x_52); +if (lean_is_exclusive(x_8)) { + lean_ctor_release(x_8, 0); + lean_ctor_release(x_8, 1); + x_53 = x_8; } else { - x_109 = x_87; -} -lean_ctor_set(x_109, 0, x_108); -x_110 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_110, 0, x_109); -lean_ctor_set(x_110, 1, x_85); -return x_110; + lean_dec_ref(x_8); + x_53 = lean_box(0); } -default: -{ -lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; -x_111 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; -x_112 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -x_113 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__13; -x_114 = l_Lean_mkApp4(x_111, x_112, x_113, x_92, x_93); -x_115 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_115, 0, x_90); -lean_ctor_set(x_115, 1, x_96); -lean_ctor_set(x_115, 2, x_114); -if (lean_is_scalar(x_87)) { - x_116 = lean_alloc_ctor(1, 1, 0); +x_54 = lean_ctor_get(x_51, 0); +lean_inc(x_54); +x_55 = lean_ctor_get(x_51, 2); +lean_inc(x_55); +x_56 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_56, 0, x_54); +x_57 = lean_box(0); +x_58 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__3; +x_59 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7; +lean_inc(x_55); +x_60 = l_Lean_mkAppB(x_58, x_59, x_55); +x_61 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___boxed), 7, 1); +lean_closure_set(x_61, 0, x_55); +lean_inc(x_51); +x_62 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__7), 10, 3); +lean_closure_set(x_62, 0, x_51); +lean_closure_set(x_62, 1, x_57); +lean_closure_set(x_62, 2, x_1); +if (lean_is_exclusive(x_51)) { + lean_ctor_release(x_51, 0); + lean_ctor_release(x_51, 1); + lean_ctor_release(x_51, 2); + x_63 = x_51; } else { - x_116 = x_87; + lean_dec_ref(x_51); + x_63 = lean_box(0); } -lean_ctor_set(x_116, 0, x_115); -x_117 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_117, 0, x_116); -lean_ctor_set(x_117, 1, x_85); -return x_117; +x_64 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_64, 0, x_61); +lean_closure_set(x_64, 1, x_62); +if (lean_is_scalar(x_63)) { + x_65 = lean_alloc_ctor(0, 3, 0); +} else { + x_65 = x_63; } +lean_ctor_set(x_65, 0, x_56); +lean_ctor_set(x_65, 1, x_64); +lean_ctor_set(x_65, 2, x_60); +x_66 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_66, 0, x_65); +if (lean_is_scalar(x_53)) { + x_67 = lean_alloc_ctor(0, 2, 0); +} else { + x_67 = x_53; } +lean_ctor_set(x_67, 0, x_66); +lean_ctor_set(x_67, 1, x_52); +return x_67; } } } else { -uint8_t x_118; -lean_dec(x_20); -lean_dec(x_4); -lean_dec(x_2); +uint8_t x_68; lean_dec(x_1); -x_118 = !lean_is_exclusive(x_21); -if (x_118 == 0) +x_68 = !lean_is_exclusive(x_8); +if (x_68 == 0) { -return x_21; +return x_8; } else { -lean_object* x_119; lean_object* x_120; lean_object* x_121; -x_119 = lean_ctor_get(x_21, 0); -x_120 = lean_ctor_get(x_21, 1); -lean_inc(x_120); -lean_inc(x_119); -lean_dec(x_21); -x_121 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_121, 0, x_119); -lean_ctor_set(x_121, 1, x_120); -return x_121; +lean_object* x_69; lean_object* x_70; lean_object* x_71; +x_69 = lean_ctor_get(x_8, 0); +x_70 = lean_ctor_get(x_8, 1); +lean_inc(x_70); +lean_inc(x_69); +lean_dec(x_8); +x_71 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_71, 0, x_69); +lean_ctor_set(x_71, 1, x_70); +return x_71; } } } } -else -{ -uint8_t x_122; -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -x_122 = !lean_is_exclusive(x_11); -if (x_122 == 0) +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__1() { +_start: { -return x_11; +uint8_t x_1; lean_object* x_2; +x_1 = 0; +x_2 = lean_alloc_ctor(1, 0, 1); +lean_ctor_set_uint8(x_2, 0, x_1); +return x_2; } -else +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__2() { +_start: { -lean_object* x_123; lean_object* x_124; lean_object* x_125; -x_123 = lean_ctor_get(x_11, 0); -x_124 = lean_ctor_get(x_11, 1); -lean_inc(x_124); -lean_inc(x_123); -lean_dec(x_11); -x_125 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_125, 0, x_123); -lean_ctor_set(x_125, 1, x_124); -return x_125; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("const", 5, 5); +return x_1; } } +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__2; +x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); +return x_6; } } -LEAN_EXPORT lean_object* l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__4() { _start: { -lean_object* x_8; -x_8 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_8, 0, x_1); -lean_ctor_set(x_8, 1, x_7); -return x_8; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__3; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; } } -LEAN_EXPORT lean_object* l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___spec__1(lean_object* x_1) { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__5() { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___spec__1___rarg___boxed), 7, 0); -return x_2; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("false", 5, 5); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__6() { _start: { -lean_object* x_9; -x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred(x_1, x_3, x_4, x_5, x_6, x_7, x_8); -return x_9; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__5; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__7() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Reflect", 7, 7); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__6; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__8() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("beq_congr", 9, 9); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__4; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__7; +x_4 = l_Lean_mkAppB(x_1, x_2, x_3); +return x_4; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__9() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__2; -x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); -return x_7; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__7; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { -uint8_t x_10; lean_object* x_11; lean_object* x_12; -x_10 = 2; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__3; -x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection(x_1, x_2, x_10, x_11, x_4, x_5, x_6, x_7, x_8, x_9); -return x_12; +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__9; +x_9 = lean_alloc_closure((void*)(l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___spec__1___rarg___boxed), 7, 1); +lean_closure_set(x_9, 0, x_8); +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__1; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__8; +x_12 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_12, 0, x_10); +lean_ctor_set(x_12, 1, x_9); +lean_ctor_set(x_12, 2, x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_12); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_13); +lean_ctor_set(x_14, 1, x_7); +return x_14; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__1() { _start: { -lean_object* x_8; lean_object* x_9; -x_8 = lean_box(0); -x_9 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_9, 0, x_8); -lean_ctor_set(x_9, 1, x_7); -return x_9; +uint8_t x_1; lean_object* x_2; +x_1 = 1; +x_2 = lean_alloc_ctor(1, 0, 1); +lean_ctor_set_uint8(x_2, 0, x_1); +return x_2; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__2() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__3___boxed), 7, 0); +x_1 = lean_mk_string_unchecked("true", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("BitVec", 6, 6); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__2; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4___closed__2; -x_3 = l_Lean_Name_str___override(x_1, x_2); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__3; +x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__5() { _start: { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; -x_11 = l_Lean_Meta_instantiateMVarsIfMVarApp(x_2, x_6, x_7, x_8, x_9, x_10); -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); -x_13 = lean_ctor_get(x_11, 1); -lean_inc(x_13); -lean_dec(x_11); -x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4___closed__1; -x_15 = l_Lean_Expr_cleanupAnnotations(x_12); -x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__8; -x_17 = l_Lean_Expr_isConstOf(x_15, x_16); -if (x_17 == 0) -{ -uint8_t x_18; -lean_dec(x_4); -lean_dec(x_3); -x_18 = l_Lean_Expr_isApp(x_15); -if (x_18 == 0) +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__4; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__4; +x_4 = l_Lean_mkAppB(x_1, x_2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__6() { +_start: { -lean_object* x_19; lean_object* x_20; -lean_dec(x_15); -lean_dec(x_1); -x_19 = lean_box(0); -x_20 = lean_apply_7(x_14, x_19, x_5, x_6, x_7, x_8, x_9, x_13); -return x_20; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__4; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl(x_1); +return x_2; } -else +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: { -lean_object* x_21; lean_object* x_22; uint8_t x_23; -x_21 = l_Lean_Expr_appFnCleanup(x_15, lean_box(0)); -x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4___closed__3; -x_23 = l_Lean_Expr_isConstOf(x_21, x_22); -lean_dec(x_21); -if (x_23 == 0) +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__6; +x_9 = lean_alloc_closure((void*)(l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___spec__1___rarg___boxed), 7, 1); +lean_closure_set(x_9, 0, x_8); +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__1; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__5; +x_12 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_12, 0, x_10); +lean_ctor_set(x_12, 1, x_9); +lean_ctor_set(x_12, 2, x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_12); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_13); +lean_ctor_set(x_14, 1, x_7); +return x_14; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__1() { +_start: { -lean_object* x_24; lean_object* x_25; -lean_dec(x_1); -x_24 = lean_box(0); -x_25 = lean_apply_7(x_14, x_24, x_5, x_6, x_7, x_8, x_9, x_13); -return x_25; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__5), 8, 0); +return x_1; } -else +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__2() { +_start: { -lean_object* x_26; -x_26 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred(x_1, x_5, x_6, x_7, x_8, x_9, x_13); -return x_26; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__6), 8, 0); +return x_1; } } +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8), 7, 0); +return x_1; +} } -else +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__4() { +_start: { -lean_object* x_27; lean_object* x_28; -lean_dec(x_15); -lean_dec(x_1); -x_27 = lean_box(0); -x_28 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2(x_3, x_4, x_27, x_5, x_6, x_7, x_8, x_9, x_13); -return x_28; -} +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___boxed), 7, 0); +return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__5___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__5() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("xor_congr", 9, 9); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___boxed), 7, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__5___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__6() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__5___closed__1; -x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); -return x_7; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__1; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__7() { _start: { -uint8_t x_9; lean_object* x_10; lean_object* x_11; -x_9 = 1; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__5___closed__2; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection(x_1, x_2, x_9, x_10, x_3, x_4, x_5, x_6, x_7, x_8); -return x_11; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("xor", 3, 3); +return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__6___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__7; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__9() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("and_congr", 9, 9); +x_1 = lean_mk_string_unchecked("and", 3, 3); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__6___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__10() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__6___closed__1; -x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); -return x_7; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__9; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__11() { _start: { -uint8_t x_9; lean_object* x_10; lean_object* x_11; -x_9 = 0; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__6___closed__2; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection(x_1, x_2, x_9, x_10, x_3, x_4, x_5, x_6, x_7, x_8); -return x_11; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("BEq", 3, 3); +return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__7___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__12() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("not_congr", 9, 9); +x_1 = lean_mk_string_unchecked("beq", 3, 3); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__7___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__13() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__7___closed__1; -x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); -return x_7; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__11; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__12; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { -lean_object* x_11; lean_object* x_12; -x_11 = lean_ctor_get(x_1, 1); -lean_inc(x_11); -lean_dec(x_1); -x_12 = lean_apply_6(x_11, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_12) == 0) +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; +lean_inc(x_1); +x_8 = l_Lean_Meta_instantiateMVarsIfMVarApp(x_1, x_3, x_4, x_5, x_6, x_7); +x_9 = lean_ctor_get(x_8, 0); +lean_inc(x_9); +x_10 = lean_ctor_get(x_8, 1); +lean_inc(x_10); +lean_dec(x_8); +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__1; +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__2; +x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__3; +x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__4; +x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__5; +x_16 = l_Lean_Expr_cleanupAnnotations(x_9); +x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__6; +x_18 = l_Lean_Expr_isConstOf(x_16, x_17); +if (x_18 == 0) { -uint8_t x_13; -x_13 = !lean_is_exclusive(x_12); -if (x_13 == 0) +lean_object* x_19; uint8_t x_20; +x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__3; +x_20 = l_Lean_Expr_isConstOf(x_16, x_19); +if (x_20 == 0) { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_14 = lean_ctor_get(x_12, 0); -x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__7___closed__2; -x_16 = l_Lean_Expr_const___override(x_15, x_2); -x_17 = l_Lean_mkApp3(x_16, x_3, x_4, x_14); -lean_ctor_set(x_12, 0, x_17); -return x_12; +uint8_t x_21; +x_21 = l_Lean_Expr_isApp(x_16); +if (x_21 == 0) +{ +lean_object* x_22; +lean_dec(x_16); +x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred(x_1, x_2, x_3, x_4, x_5, x_6, x_10); +return x_22; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_18 = lean_ctor_get(x_12, 0); -x_19 = lean_ctor_get(x_12, 1); -lean_inc(x_19); -lean_inc(x_18); -lean_dec(x_12); -x_20 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__7___closed__2; -x_21 = l_Lean_Expr_const___override(x_20, x_2); -x_22 = l_Lean_mkApp3(x_21, x_3, x_4, x_18); -x_23 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_23, 0, x_22); -lean_ctor_set(x_23, 1, x_19); -return x_23; +lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; +x_23 = l_Lean_Expr_appArg(x_16, lean_box(0)); +x_24 = l_Lean_Expr_appFnCleanup(x_16, lean_box(0)); +x_25 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__6; +x_26 = l_Lean_Expr_isConstOf(x_24, x_25); +if (x_26 == 0) +{ +uint8_t x_27; +x_27 = l_Lean_Expr_isApp(x_24); +if (x_27 == 0) +{ +lean_object* x_28; +lean_dec(x_24); +lean_dec(x_23); +x_28 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred(x_1, x_2, x_3, x_4, x_5, x_6, x_10); +return x_28; } +else +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; +x_29 = l_Lean_Expr_appArg(x_24, lean_box(0)); +x_30 = l_Lean_Expr_appFnCleanup(x_24, lean_box(0)); +x_31 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__8; +x_32 = l_Lean_Expr_isConstOf(x_30, x_31); +if (x_32 == 0) +{ +lean_object* x_33; uint8_t x_34; +x_33 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__10; +x_34 = l_Lean_Expr_isConstOf(x_30, x_33); +if (x_34 == 0) +{ +uint8_t x_35; +x_35 = l_Lean_Expr_isApp(x_30); +if (x_35 == 0) +{ +lean_object* x_36; +lean_dec(x_30); +lean_dec(x_29); +lean_dec(x_23); +x_36 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred(x_1, x_2, x_3, x_4, x_5, x_6, x_10); +return x_36; } else { -uint8_t x_24; -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_24 = !lean_is_exclusive(x_12); -if (x_24 == 0) +lean_object* x_37; uint8_t x_38; +x_37 = l_Lean_Expr_appFnCleanup(x_30, lean_box(0)); +x_38 = l_Lean_Expr_isApp(x_37); +if (x_38 == 0) { -return x_12; +lean_object* x_39; +lean_dec(x_37); +lean_dec(x_29); +lean_dec(x_23); +x_39 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred(x_1, x_2, x_3, x_4, x_5, x_6, x_10); +return x_39; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_12, 0); -x_26 = lean_ctor_get(x_12, 1); -lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_12); -x_27 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_26); -return x_27; +lean_object* x_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; +x_40 = l_Lean_Expr_appArg(x_37, lean_box(0)); +x_41 = l_Lean_Expr_appFnCleanup(x_37, lean_box(0)); +x_42 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__13; +x_43 = l_Lean_Expr_isConstOf(x_41, x_42); +lean_dec(x_41); +if (x_43 == 0) +{ +lean_object* x_44; +lean_dec(x_40); +lean_dec(x_29); +lean_dec(x_23); +x_44 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred(x_1, x_2, x_3, x_4, x_5, x_6, x_10); +return x_44; +} +else +{ +lean_object* x_45; +x_45 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4(x_1, x_40, x_29, x_23, x_2, x_3, x_4, x_5, x_6, x_10); +return x_45; } } } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("not", 3, 3); -return x_1; +lean_object* x_46; +lean_dec(x_30); +lean_dec(x_1); +x_46 = lean_apply_8(x_12, x_29, x_23, x_2, x_3, x_4, x_5, x_6, x_10); +return x_46; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__2() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__1; -x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); -return x_6; +lean_object* x_47; +lean_dec(x_30); +lean_dec(x_1); +x_47 = lean_apply_8(x_11, x_29, x_23, x_2, x_3, x_4, x_5, x_6, x_10); +return x_47; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__3() { -_start: +} +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__2; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; +lean_object* x_48; +lean_dec(x_24); +lean_dec(x_1); +x_48 = lean_apply_7(x_13, x_23, x_2, x_3, x_4, x_5, x_6, x_10); +return x_48; +} +} +} +else +{ +lean_object* x_49; lean_object* x_50; +lean_dec(x_16); +lean_dec(x_1); +x_49 = lean_box(0); +x_50 = lean_apply_7(x_15, x_49, x_2, x_3, x_4, x_5, x_6, x_10); +return x_50; +} +} +else +{ +lean_object* x_51; lean_object* x_52; +lean_dec(x_16); +lean_dec(x_1); +x_51 = lean_box(0); +x_52 = lean_apply_7(x_14, x_51, x_2, x_3, x_4, x_5, x_6, x_10); +return x_52; +} } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goOrAtom(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); lean_inc(x_1); -x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go(x_1, x_2, x_3, x_4, x_5, x_6, x_7); if (lean_obj_tag(x_8) == 0) { lean_object* x_9; @@ -1723,701 +1790,785 @@ x_9 = lean_ctor_get(x_8, 0); lean_inc(x_9); if (lean_obj_tag(x_9) == 0) { -uint8_t x_10; -lean_dec(x_1); -x_10 = !lean_is_exclusive(x_8); -if (x_10 == 0) -{ -lean_object* x_11; lean_object* x_12; -x_11 = lean_ctor_get(x_8, 0); -lean_dec(x_11); -x_12 = lean_box(0); -lean_ctor_set(x_8, 0, x_12); -return x_8; -} -else -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_ctor_get(x_8, 1); -lean_inc(x_13); +lean_object* x_10; lean_object* x_11; +x_10 = lean_ctor_get(x_8, 1); +lean_inc(x_10); lean_dec(x_8); -x_14 = lean_box(0); -x_15 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_15, 0, x_14); -lean_ctor_set(x_15, 1, x_13); -return x_15; -} +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_boolAtom(x_1, x_2, x_3, x_4, x_5, x_6, x_10); +return x_11; } else { -uint8_t x_16; -x_16 = !lean_is_exclusive(x_9); -if (x_16 == 0) -{ -uint8_t x_17; -x_17 = !lean_is_exclusive(x_8); -if (x_17 == 0) +uint8_t x_12; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_12 = !lean_is_exclusive(x_8); +if (x_12 == 0) { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; -x_18 = lean_ctor_get(x_9, 0); -x_19 = lean_ctor_get(x_8, 0); -lean_dec(x_19); -x_20 = lean_ctor_get(x_18, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_18, 2); -lean_inc(x_21); -x_22 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_22, 0, x_20); -x_23 = lean_box(0); -x_24 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__3; -x_25 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -lean_inc(x_21); -x_26 = l_Lean_mkAppB(x_24, x_25, x_21); -x_27 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___boxed), 7, 1); -lean_closure_set(x_27, 0, x_21); -lean_inc(x_18); -x_28 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__7), 10, 3); -lean_closure_set(x_28, 0, x_18); -lean_closure_set(x_28, 1, x_23); -lean_closure_set(x_28, 2, x_1); -x_29 = !lean_is_exclusive(x_18); -if (x_29 == 0) +lean_object* x_13; uint8_t x_14; +x_13 = lean_ctor_get(x_8, 0); +lean_dec(x_13); +x_14 = !lean_is_exclusive(x_9); +if (x_14 == 0) { -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_30 = lean_ctor_get(x_18, 2); -lean_dec(x_30); -x_31 = lean_ctor_get(x_18, 1); -lean_dec(x_31); -x_32 = lean_ctor_get(x_18, 0); -lean_dec(x_32); -x_33 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_33, 0, x_27); -lean_closure_set(x_33, 1, x_28); -lean_ctor_set(x_18, 2, x_26); -lean_ctor_set(x_18, 1, x_33); -lean_ctor_set(x_18, 0, x_22); return x_8; } else { -lean_object* x_34; lean_object* x_35; -lean_dec(x_18); -x_34 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_34, 0, x_27); -lean_closure_set(x_34, 1, x_28); -x_35 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_35, 0, x_22); -lean_ctor_set(x_35, 1, x_34); -lean_ctor_set(x_35, 2, x_26); -lean_ctor_set(x_9, 0, x_35); +lean_object* x_15; lean_object* x_16; +x_15 = lean_ctor_get(x_9, 0); +lean_inc(x_15); +lean_dec(x_9); +x_16 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_8, 0, x_16); return x_8; } } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_36 = lean_ctor_get(x_9, 0); -x_37 = lean_ctor_get(x_8, 1); -lean_inc(x_37); +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_17 = lean_ctor_get(x_8, 1); +lean_inc(x_17); lean_dec(x_8); -x_38 = lean_ctor_get(x_36, 0); -lean_inc(x_38); -x_39 = lean_ctor_get(x_36, 2); -lean_inc(x_39); -x_40 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_40, 0, x_38); -x_41 = lean_box(0); -x_42 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__3; -x_43 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -lean_inc(x_39); -x_44 = l_Lean_mkAppB(x_42, x_43, x_39); -x_45 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___boxed), 7, 1); -lean_closure_set(x_45, 0, x_39); -lean_inc(x_36); -x_46 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__7), 10, 3); -lean_closure_set(x_46, 0, x_36); -lean_closure_set(x_46, 1, x_41); -lean_closure_set(x_46, 2, x_1); -if (lean_is_exclusive(x_36)) { - lean_ctor_release(x_36, 0); - lean_ctor_release(x_36, 1); - lean_ctor_release(x_36, 2); - x_47 = x_36; +x_18 = lean_ctor_get(x_9, 0); +lean_inc(x_18); +if (lean_is_exclusive(x_9)) { + lean_ctor_release(x_9, 0); + x_19 = x_9; } else { - lean_dec_ref(x_36); - x_47 = lean_box(0); + lean_dec_ref(x_9); + x_19 = lean_box(0); } -x_48 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_48, 0, x_45); -lean_closure_set(x_48, 1, x_46); -if (lean_is_scalar(x_47)) { - x_49 = lean_alloc_ctor(0, 3, 0); +if (lean_is_scalar(x_19)) { + x_20 = lean_alloc_ctor(1, 1, 0); } else { - x_49 = x_47; + x_20 = x_19; +} +lean_ctor_set(x_20, 0, x_18); +x_21 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_21, 0, x_20); +lean_ctor_set(x_21, 1, x_17); +return x_21; } -lean_ctor_set(x_49, 0, x_40); -lean_ctor_set(x_49, 1, x_48); -lean_ctor_set(x_49, 2, x_44); -lean_ctor_set(x_9, 0, x_49); -x_50 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_50, 0, x_9); -lean_ctor_set(x_50, 1, x_37); -return x_50; } } else { -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; -x_51 = lean_ctor_get(x_9, 0); -lean_inc(x_51); -lean_dec(x_9); -x_52 = lean_ctor_get(x_8, 1); -lean_inc(x_52); -if (lean_is_exclusive(x_8)) { - lean_ctor_release(x_8, 0); - lean_ctor_release(x_8, 1); - x_53 = x_8; -} else { - lean_dec_ref(x_8); - x_53 = lean_box(0); +uint8_t x_22; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_22 = !lean_is_exclusive(x_8); +if (x_22 == 0) +{ +return x_8; } -x_54 = lean_ctor_get(x_51, 0); -lean_inc(x_54); -x_55 = lean_ctor_get(x_51, 2); -lean_inc(x_55); -x_56 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_56, 0, x_54); -x_57 = lean_box(0); -x_58 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__3; -x_59 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -lean_inc(x_55); -x_60 = l_Lean_mkAppB(x_58, x_59, x_55); -x_61 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___boxed), 7, 1); -lean_closure_set(x_61, 0, x_55); -lean_inc(x_51); -x_62 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__7), 10, 3); -lean_closure_set(x_62, 0, x_51); -lean_closure_set(x_62, 1, x_57); -lean_closure_set(x_62, 2, x_1); -if (lean_is_exclusive(x_51)) { - lean_ctor_release(x_51, 0); - lean_ctor_release(x_51, 1); - lean_ctor_release(x_51, 2); - x_63 = x_51; -} else { - lean_dec_ref(x_51); - x_63 = lean_box(0); +else +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_8, 0); +x_24 = lean_ctor_get(x_8, 1); +lean_inc(x_24); +lean_inc(x_23); +lean_dec(x_8); +x_25 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +return x_25; } -x_64 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_64, 0, x_61); -lean_closure_set(x_64, 1, x_62); -if (lean_is_scalar(x_63)) { - x_65 = lean_alloc_ctor(0, 3, 0); -} else { - x_65 = x_63; } -lean_ctor_set(x_65, 0, x_56); -lean_ctor_set(x_65, 1, x_64); -lean_ctor_set(x_65, 2, x_60); -x_66 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_66, 0, x_65); -if (lean_is_scalar(x_53)) { - x_67 = lean_alloc_ctor(0, 2, 0); -} else { - x_67 = x_53; } -lean_ctor_set(x_67, 0, x_66); -lean_ctor_set(x_67, 1, x_52); -return x_67; } +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr(x_1, x_9, x_10, x_11, x_12, x_13, x_14); +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_15, 1); +lean_inc(x_17); +lean_dec(x_15); +x_18 = lean_ctor_get(x_2, 1); +lean_inc(x_18); +lean_dec(x_2); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +x_19 = lean_apply_6(x_18, x_9, x_10, x_11, x_12, x_13, x_17); +if (lean_obj_tag(x_19) == 0) +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_19, 1); +lean_inc(x_21); +lean_dec(x_19); +x_22 = lean_ctor_get(x_3, 1); +lean_inc(x_22); +lean_dec(x_3); +x_23 = lean_apply_6(x_22, x_9, x_10, x_11, x_12, x_13, x_21); +if (lean_obj_tag(x_23) == 0) +{ +uint8_t x_24; +x_24 = !lean_is_exclusive(x_23); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_23, 0); +x_26 = l_Lean_Expr_const___override(x_4, x_5); +x_27 = l_Lean_mkApp6(x_26, x_6, x_7, x_8, x_16, x_20, x_25); +lean_ctor_set(x_23, 0, x_27); +return x_23; +} +else +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_28 = lean_ctor_get(x_23, 0); +x_29 = lean_ctor_get(x_23, 1); +lean_inc(x_29); +lean_inc(x_28); +lean_dec(x_23); +x_30 = l_Lean_Expr_const___override(x_4, x_5); +x_31 = l_Lean_mkApp6(x_30, x_6, x_7, x_8, x_16, x_20, x_28); +x_32 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_32, 0, x_31); +lean_ctor_set(x_32, 1, x_29); +return x_32; } } else { -uint8_t x_68; -lean_dec(x_1); -x_68 = !lean_is_exclusive(x_8); -if (x_68 == 0) +uint8_t x_33; +lean_dec(x_20); +lean_dec(x_16); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_33 = !lean_is_exclusive(x_23); +if (x_33 == 0) { -return x_8; +return x_23; } else { -lean_object* x_69; lean_object* x_70; lean_object* x_71; -x_69 = lean_ctor_get(x_8, 0); -x_70 = lean_ctor_get(x_8, 1); -lean_inc(x_70); -lean_inc(x_69); -lean_dec(x_8); -x_71 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_71, 0, x_69); -lean_ctor_set(x_71, 1, x_70); -return x_71; +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_23, 0); +x_35 = lean_ctor_get(x_23, 1); +lean_inc(x_35); +lean_inc(x_34); +lean_dec(x_23); +x_36 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_36, 0, x_34); +lean_ctor_set(x_36, 1, x_35); +return x_36; } } } +else +{ +uint8_t x_37; +lean_dec(x_16); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_37 = !lean_is_exclusive(x_19); +if (x_37 == 0) +{ +return x_19; } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__1() { -_start: +else { -uint8_t x_1; lean_object* x_2; -x_1 = 0; -x_2 = lean_alloc_ctor(1, 0, 1); -lean_ctor_set_uint8(x_2, 0, x_1); -return x_2; +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_19, 0); +x_39 = lean_ctor_get(x_19, 1); +lean_inc(x_39); +lean_inc(x_38); +lean_dec(x_19); +x_40 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +return x_40; +} } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__2() { +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("const", 5, 5); +x_1 = lean_mk_string_unchecked("gate", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__2; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__1; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__3; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__2; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__4() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("false", 5, 5); +x_1 = lean_mk_string_unchecked("Gate", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__6() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__5() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__5; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__4; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__9; +x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); +return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__7() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__6; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__5; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__8() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__4; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__7; -x_4 = l_Lean_mkAppB(x_1, x_2, x_3); -return x_4; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__9() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__7; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__9; -x_9 = lean_alloc_closure((void*)(l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___spec__1___rarg___boxed), 7, 1); -lean_closure_set(x_9, 0, x_8); -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__1; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__8; -x_12 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_12, 0, x_10); -lean_ctor_set(x_12, 1, x_9); -lean_ctor_set(x_12, 2, x_11); -x_13 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_13, 0, x_12); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_13); -lean_ctor_set(x_14, 1, x_7); -return x_14; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__1() { -_start: -{ -uint8_t x_1; lean_object* x_2; -x_1 = 1; -x_2 = lean_alloc_ctor(1, 0, 1); -lean_ctor_set_uint8(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__2() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("true", 4, 4); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__7() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__2; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__4; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__7; +x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); +return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__3; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__7; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__4; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__4; -x_4 = l_Lean_mkAppB(x_1, x_2, x_3); -return x_4; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__4; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__6; -x_9 = lean_alloc_closure((void*)(l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___spec__1___rarg___boxed), 7, 1); -lean_closure_set(x_9, 0, x_8); -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__1; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__5; -x_12 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_12, 0, x_10); -lean_ctor_set(x_12, 1, x_9); -lean_ctor_set(x_12, 2, x_11); -x_13 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_13, 0, x_12); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_13); -lean_ctor_set(x_14, 1, x_7); -return x_14; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__5), 8, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__2() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__6), 8, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8), 7, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___boxed), 7, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__5() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___boxed), 7, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__1; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__7() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__8; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__8() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__5; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__9() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__9() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("BEq", 3, 3); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__4; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__12; +x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); +return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__10() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__9; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__11; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__9; +x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; -lean_inc(x_1); -x_8 = l_Lean_Meta_instantiateMVarsIfMVarApp(x_1, x_3, x_4, x_5, x_6, x_7); -x_9 = lean_ctor_get(x_8, 0); +lean_object* x_11; lean_inc(x_9); -x_10 = lean_ctor_get(x_8, 1); -lean_inc(x_10); -lean_dec(x_8); -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__1; -x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__2; -x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__3; -x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__4; -x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__5; -x_16 = l_Lean_Expr_cleanupAnnotations(x_9); -x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__6; -x_18 = l_Lean_Expr_isConstOf(x_16, x_17); -if (x_18 == 0) +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_1); +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goOrAtom(x_1, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_11) == 0) { -lean_object* x_19; uint8_t x_20; -x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__3; -x_20 = l_Lean_Expr_isConstOf(x_16, x_19); -if (x_20 == 0) +lean_object* x_12; +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +if (lean_obj_tag(x_12) == 0) { -uint8_t x_21; -x_21 = l_Lean_Expr_isApp(x_16); -if (x_21 == 0) +uint8_t x_13; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_13 = !lean_is_exclusive(x_11); +if (x_13 == 0) { -lean_object* x_22; -lean_dec(x_16); -x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred(x_1, x_2, x_3, x_4, x_5, x_6, x_10); -return x_22; +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_11, 0); +lean_dec(x_14); +x_15 = lean_box(0); +lean_ctor_set(x_11, 0, x_15); +return x_11; } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; -x_23 = l_Lean_Expr_appArg(x_16, lean_box(0)); -x_24 = l_Lean_Expr_appFnCleanup(x_16, lean_box(0)); -x_25 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__6; -x_26 = l_Lean_Expr_isConstOf(x_24, x_25); -if (x_26 == 0) +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_11, 1); +lean_inc(x_16); +lean_dec(x_11); +x_17 = lean_box(0); +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set(x_18, 1, x_16); +return x_18; +} +} +else { -uint8_t x_27; -x_27 = l_Lean_Expr_isApp(x_24); -if (x_27 == 0) +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_11, 1); +lean_inc(x_19); +lean_dec(x_11); +x_20 = lean_ctor_get(x_12, 0); +lean_inc(x_20); +lean_dec(x_12); +lean_inc(x_2); +x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goOrAtom(x_2, x_5, x_6, x_7, x_8, x_9, x_19); +if (lean_obj_tag(x_21) == 0) { -lean_object* x_28; +lean_object* x_22; +x_22 = lean_ctor_get(x_21, 0); +lean_inc(x_22); +if (lean_obj_tag(x_22) == 0) +{ +uint8_t x_23; +lean_dec(x_20); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_23 = !lean_is_exclusive(x_21); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_21, 0); lean_dec(x_24); -lean_dec(x_23); -x_28 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred(x_1, x_2, x_3, x_4, x_5, x_6, x_10); +x_25 = lean_box(0); +lean_ctor_set(x_21, 0, x_25); +return x_21; +} +else +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_21, 1); +lean_inc(x_26); +lean_dec(x_21); +x_27 = lean_box(0); +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_26); return x_28; } +} else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; -x_29 = l_Lean_Expr_appArg(x_24, lean_box(0)); -x_30 = l_Lean_Expr_appFnCleanup(x_24, lean_box(0)); -x_31 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__7; -x_32 = l_Lean_Expr_isConstOf(x_30, x_31); -if (x_32 == 0) +uint8_t x_29; +x_29 = !lean_is_exclusive(x_21); +if (x_29 == 0) { -lean_object* x_33; uint8_t x_34; -x_33 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__8; -x_34 = l_Lean_Expr_isConstOf(x_30, x_33); -if (x_34 == 0) +lean_object* x_30; uint8_t x_31; +x_30 = lean_ctor_get(x_21, 0); +lean_dec(x_30); +x_31 = !lean_is_exclusive(x_22); +if (x_31 == 0) +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_32 = lean_ctor_get(x_22, 0); +x_33 = lean_ctor_get(x_20, 0); +lean_inc(x_33); +x_34 = lean_ctor_get(x_32, 0); +lean_inc(x_34); +x_35 = lean_alloc_ctor(3, 2, 1); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +lean_ctor_set_uint8(x_35, sizeof(void*)*2, x_3); +x_36 = lean_box(0); +x_37 = lean_ctor_get(x_20, 2); +lean_inc(x_37); +x_38 = lean_ctor_get(x_32, 2); +lean_inc(x_38); +lean_inc(x_37); +x_39 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___boxed), 7, 1); +lean_closure_set(x_39, 0, x_37); +lean_inc(x_38); +x_40 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___lambda__1), 14, 7); +lean_closure_set(x_40, 0, x_38); +lean_closure_set(x_40, 1, x_20); +lean_closure_set(x_40, 2, x_32); +lean_closure_set(x_40, 3, x_4); +lean_closure_set(x_40, 4, x_36); +lean_closure_set(x_40, 5, x_1); +lean_closure_set(x_40, 6, x_2); +x_41 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_41, 0, x_39); +lean_closure_set(x_41, 1, x_40); +switch (x_3) { +case 0: +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_42 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; +x_43 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7; +x_44 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__6; +x_45 = l_Lean_mkApp4(x_42, x_43, x_44, x_37, x_38); +x_46 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_46, 0, x_35); +lean_ctor_set(x_46, 1, x_41); +lean_ctor_set(x_46, 2, x_45); +lean_ctor_set(x_22, 0, x_46); +return x_21; +} +case 1: +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_47 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; +x_48 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7; +x_49 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__8; +x_50 = l_Lean_mkApp4(x_47, x_48, x_49, x_37, x_38); +x_51 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_51, 0, x_35); +lean_ctor_set(x_51, 1, x_41); +lean_ctor_set(x_51, 2, x_50); +lean_ctor_set(x_22, 0, x_51); +return x_21; +} +default: +{ +lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; +x_52 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; +x_53 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7; +x_54 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__10; +x_55 = l_Lean_mkApp4(x_52, x_53, x_54, x_37, x_38); +x_56 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_56, 0, x_35); +lean_ctor_set(x_56, 1, x_41); +lean_ctor_set(x_56, 2, x_55); +lean_ctor_set(x_22, 0, x_56); +return x_21; +} +} +} +else +{ +lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; +x_57 = lean_ctor_get(x_22, 0); +lean_inc(x_57); +lean_dec(x_22); +x_58 = lean_ctor_get(x_20, 0); +lean_inc(x_58); +x_59 = lean_ctor_get(x_57, 0); +lean_inc(x_59); +x_60 = lean_alloc_ctor(3, 2, 1); +lean_ctor_set(x_60, 0, x_58); +lean_ctor_set(x_60, 1, x_59); +lean_ctor_set_uint8(x_60, sizeof(void*)*2, x_3); +x_61 = lean_box(0); +x_62 = lean_ctor_get(x_20, 2); +lean_inc(x_62); +x_63 = lean_ctor_get(x_57, 2); +lean_inc(x_63); +lean_inc(x_62); +x_64 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___boxed), 7, 1); +lean_closure_set(x_64, 0, x_62); +lean_inc(x_63); +x_65 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___lambda__1), 14, 7); +lean_closure_set(x_65, 0, x_63); +lean_closure_set(x_65, 1, x_20); +lean_closure_set(x_65, 2, x_57); +lean_closure_set(x_65, 3, x_4); +lean_closure_set(x_65, 4, x_61); +lean_closure_set(x_65, 5, x_1); +lean_closure_set(x_65, 6, x_2); +x_66 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_66, 0, x_64); +lean_closure_set(x_66, 1, x_65); +switch (x_3) { +case 0: +{ +lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; +x_67 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; +x_68 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7; +x_69 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__6; +x_70 = l_Lean_mkApp4(x_67, x_68, x_69, x_62, x_63); +x_71 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_71, 0, x_60); +lean_ctor_set(x_71, 1, x_66); +lean_ctor_set(x_71, 2, x_70); +x_72 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_72, 0, x_71); +lean_ctor_set(x_21, 0, x_72); +return x_21; +} +case 1: { -uint8_t x_35; -x_35 = l_Lean_Expr_isApp(x_30); -if (x_35 == 0) +lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; +x_73 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; +x_74 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7; +x_75 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__8; +x_76 = l_Lean_mkApp4(x_73, x_74, x_75, x_62, x_63); +x_77 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_77, 0, x_60); +lean_ctor_set(x_77, 1, x_66); +lean_ctor_set(x_77, 2, x_76); +x_78 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_78, 0, x_77); +lean_ctor_set(x_21, 0, x_78); +return x_21; +} +default: { -lean_object* x_36; -lean_dec(x_30); -lean_dec(x_29); -lean_dec(x_23); -x_36 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred(x_1, x_2, x_3, x_4, x_5, x_6, x_10); -return x_36; +lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; +x_79 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; +x_80 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7; +x_81 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__10; +x_82 = l_Lean_mkApp4(x_79, x_80, x_81, x_62, x_63); +x_83 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_83, 0, x_60); +lean_ctor_set(x_83, 1, x_66); +lean_ctor_set(x_83, 2, x_82); +x_84 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_84, 0, x_83); +lean_ctor_set(x_21, 0, x_84); +return x_21; +} +} +} } else { -lean_object* x_37; uint8_t x_38; -x_37 = l_Lean_Expr_appFnCleanup(x_30, lean_box(0)); -x_38 = l_Lean_Expr_isApp(x_37); -if (x_38 == 0) -{ -lean_object* x_39; -lean_dec(x_37); -lean_dec(x_29); -lean_dec(x_23); -x_39 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred(x_1, x_2, x_3, x_4, x_5, x_6, x_10); -return x_39; +lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; +x_85 = lean_ctor_get(x_21, 1); +lean_inc(x_85); +lean_dec(x_21); +x_86 = lean_ctor_get(x_22, 0); +lean_inc(x_86); +if (lean_is_exclusive(x_22)) { + lean_ctor_release(x_22, 0); + x_87 = x_22; +} else { + lean_dec_ref(x_22); + x_87 = lean_box(0); } -else +x_88 = lean_ctor_get(x_20, 0); +lean_inc(x_88); +x_89 = lean_ctor_get(x_86, 0); +lean_inc(x_89); +x_90 = lean_alloc_ctor(3, 2, 1); +lean_ctor_set(x_90, 0, x_88); +lean_ctor_set(x_90, 1, x_89); +lean_ctor_set_uint8(x_90, sizeof(void*)*2, x_3); +x_91 = lean_box(0); +x_92 = lean_ctor_get(x_20, 2); +lean_inc(x_92); +x_93 = lean_ctor_get(x_86, 2); +lean_inc(x_93); +lean_inc(x_92); +x_94 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___boxed), 7, 1); +lean_closure_set(x_94, 0, x_92); +lean_inc(x_93); +x_95 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___lambda__1), 14, 7); +lean_closure_set(x_95, 0, x_93); +lean_closure_set(x_95, 1, x_20); +lean_closure_set(x_95, 2, x_86); +lean_closure_set(x_95, 3, x_4); +lean_closure_set(x_95, 4, x_91); +lean_closure_set(x_95, 5, x_1); +lean_closure_set(x_95, 6, x_2); +x_96 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_96, 0, x_94); +lean_closure_set(x_96, 1, x_95); +switch (x_3) { +case 0: { -lean_object* x_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; -x_40 = l_Lean_Expr_appArg(x_37, lean_box(0)); -x_41 = l_Lean_Expr_appFnCleanup(x_37, lean_box(0)); -x_42 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__10; -x_43 = l_Lean_Expr_isConstOf(x_41, x_42); -lean_dec(x_41); -if (x_43 == 0) +lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; +x_97 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; +x_98 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7; +x_99 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__6; +x_100 = l_Lean_mkApp4(x_97, x_98, x_99, x_92, x_93); +x_101 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_101, 0, x_90); +lean_ctor_set(x_101, 1, x_96); +lean_ctor_set(x_101, 2, x_100); +if (lean_is_scalar(x_87)) { + x_102 = lean_alloc_ctor(1, 1, 0); +} else { + x_102 = x_87; +} +lean_ctor_set(x_102, 0, x_101); +x_103 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_103, 0, x_102); +lean_ctor_set(x_103, 1, x_85); +return x_103; +} +case 1: { -lean_object* x_44; -lean_dec(x_40); -lean_dec(x_29); -lean_dec(x_23); -x_44 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred(x_1, x_2, x_3, x_4, x_5, x_6, x_10); -return x_44; +lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; +x_104 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; +x_105 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7; +x_106 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__8; +x_107 = l_Lean_mkApp4(x_104, x_105, x_106, x_92, x_93); +x_108 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_108, 0, x_90); +lean_ctor_set(x_108, 1, x_96); +lean_ctor_set(x_108, 2, x_107); +if (lean_is_scalar(x_87)) { + x_109 = lean_alloc_ctor(1, 1, 0); +} else { + x_109 = x_87; } -else +lean_ctor_set(x_109, 0, x_108); +x_110 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_110, 0, x_109); +lean_ctor_set(x_110, 1, x_85); +return x_110; +} +default: { -lean_object* x_45; -x_45 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4(x_1, x_40, x_29, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_45; +lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; +x_111 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; +x_112 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7; +x_113 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__10; +x_114 = l_Lean_mkApp4(x_111, x_112, x_113, x_92, x_93); +x_115 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_115, 0, x_90); +lean_ctor_set(x_115, 1, x_96); +lean_ctor_set(x_115, 2, x_114); +if (lean_is_scalar(x_87)) { + x_116 = lean_alloc_ctor(1, 1, 0); +} else { + x_116 = x_87; } +lean_ctor_set(x_116, 0, x_115); +x_117 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_117, 0, x_116); +lean_ctor_set(x_117, 1, x_85); +return x_117; } } } -else -{ -lean_object* x_46; -lean_dec(x_30); -lean_dec(x_1); -x_46 = lean_apply_8(x_12, x_29, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_46; } } else { -lean_object* x_47; -lean_dec(x_30); +uint8_t x_118; +lean_dec(x_20); +lean_dec(x_4); +lean_dec(x_2); lean_dec(x_1); -x_47 = lean_apply_8(x_11, x_29, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_47; -} -} +x_118 = !lean_is_exclusive(x_21); +if (x_118 == 0) +{ +return x_21; } else { -lean_object* x_48; -lean_dec(x_24); -lean_dec(x_1); -x_48 = lean_apply_7(x_13, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_48; +lean_object* x_119; lean_object* x_120; lean_object* x_121; +x_119 = lean_ctor_get(x_21, 0); +x_120 = lean_ctor_get(x_21, 1); +lean_inc(x_120); +lean_inc(x_119); +lean_dec(x_21); +x_121 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_121, 0, x_119); +lean_ctor_set(x_121, 1, x_120); +return x_121; +} } } } else { -lean_object* x_49; lean_object* x_50; -lean_dec(x_16); +uint8_t x_122; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); lean_dec(x_1); -x_49 = lean_box(0); -x_50 = lean_apply_7(x_15, x_49, x_2, x_3, x_4, x_5, x_6, x_10); -return x_50; -} +x_122 = !lean_is_exclusive(x_11); +if (x_122 == 0) +{ +return x_11; } else { -lean_object* x_51; lean_object* x_52; -lean_dec(x_16); -lean_dec(x_1); -x_51 = lean_box(0); -x_52 = lean_apply_7(x_14, x_51, x_2, x_3, x_4, x_5, x_6, x_10); -return x_52; -} +lean_object* x_123; lean_object* x_124; lean_object* x_125; +x_123 = lean_ctor_get(x_11, 0); +x_124 = lean_ctor_get(x_11, 1); +lean_inc(x_124); +lean_inc(x_123); +lean_dec(x_11); +x_125 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_125, 0, x_123); +lean_ctor_set(x_125, 1, x_124); +return x_125; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -uint8_t x_11; lean_object* x_12; -x_11 = lean_unbox(x_3); -lean_dec(x_3); -x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection(x_1, x_2, x_11, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_12; } } -LEAN_EXPORT lean_object* l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; -x_8 = l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); @@ -2426,29 +2577,29 @@ lean_dec(x_2); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; -x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_2); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { lean_object* x_10; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_3); return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; -x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); @@ -2458,11 +2609,11 @@ lean_dec(x_1); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; -x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); @@ -2472,11 +2623,11 @@ lean_dec(x_1); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; -x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); @@ -2486,6 +2637,24 @@ lean_dec(x_1); return x_8; } } +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +uint8_t x_11; lean_object* x_12; +x_11 = lean_unbox(x_3); +lean_dec(x_3); +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection(x_1, x_2, x_11, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; +x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goOrAtom(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +return x_8; +} +} lean_object* initialize_Lean_Elab_Tactic_BVDecide_Frontend_BVDecide_ReifiedBVPred(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Lean_Elab_Tactic_BVDecide_Frontend_BVDecide_ReifiedBVLogical(uint8_t builtin, lean_object* w) { @@ -2533,20 +2702,106 @@ l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__6 = _ lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__6); l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__7(); lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__7); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__6); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__5___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__5___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__5___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__5___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__5___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__5___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__6___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__6___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__6___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__6___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__6___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__6___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__7___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__7___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__7___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__7___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__7___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__7___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__7); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__8(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__8); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__9 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__9(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__9); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__7); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__8(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__8); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__9 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__9(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__9); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__10 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__10(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__10); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__11 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__11(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__11); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__12 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__12(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__12); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__13 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__13(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__13); l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__1(); lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__1); l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__2(); @@ -2567,92 +2822,6 @@ l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__9); l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__10 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__10(); lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__10); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__11 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__11(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__11); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__12 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__12(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__12); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__13 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__13(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__13); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__5___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__5___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__5___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__5___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__5___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__5___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__6___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__6___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__6___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__6___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__6___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__6___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__7___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__7___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__7___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__7___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__7___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__7___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__6); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__7); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__8(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__8); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__9 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__9(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__9); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__6); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__6); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__7); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__8(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__8); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__9 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__9(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__9); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__10 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__10(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__10); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/ReifiedBVPred.c b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/ReifiedBVPred.c index 546ecc9e5684..145557895eb5 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/ReifiedBVPred.c +++ b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/ReifiedBVPred.c @@ -14,219 +14,93 @@ extern "C" { #endif lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkNatLit(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__12; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__6; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__8; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__5; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__6; lean_object* l_Lean_Meta_getNatValue_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__9; lean_object* l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkApp7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__6; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__2; uint8_t l_Lean_Expr_isApp(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__10; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__3___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__3; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__4___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__6___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__3___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__1; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__8; lean_object* l_Lean_Name_mkStr5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_cleanupAnnotations(lean_object*); lean_object* l_Lean_mkApp4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__13; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__8; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__5; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__5; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__3; lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__4; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__8; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__3; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__7; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__5; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__2; lean_object* l_Lean_Expr_appArg(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__3___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_appFnCleanup(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__7; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__4; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__5; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__7; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__9; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__5___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__6___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__4___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__7; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_app___override(lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); lean_object* l_Lean_mkApp3(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__7___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__2; uint8_t l_Lean_Expr_isConstOf(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__3___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_instantiateMVarsIfMVarApp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__11; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__4___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__5; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__3; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__14; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__2___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__7___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__1___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__6; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__4___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkApp5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__4; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__7; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__6; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__6; lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: -{ -lean_object* x_17; -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -x_17 = lean_apply_6(x_1, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_17) == 0) -{ -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_17, 1); -lean_inc(x_19); -lean_dec(x_17); -x_20 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr(x_2, x_3, x_11, x_12, x_13, x_14, x_15, x_19); -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_20, 1); -lean_inc(x_22); -lean_dec(x_20); -x_23 = lean_ctor_get(x_4, 2); -lean_inc(x_23); -lean_dec(x_4); -x_24 = lean_apply_6(x_23, x_11, x_12, x_13, x_14, x_15, x_22); -if (lean_obj_tag(x_24) == 0) -{ -uint8_t x_25; -x_25 = !lean_is_exclusive(x_24); -if (x_25 == 0) -{ -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_24, 0); -x_27 = l_Lean_Expr_const___override(x_5, x_6); -x_28 = l_Lean_mkApp7(x_27, x_7, x_8, x_9, x_10, x_21, x_18, x_26); -lean_ctor_set(x_24, 0, x_28); -return x_24; -} -else -{ -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_29 = lean_ctor_get(x_24, 0); -x_30 = lean_ctor_get(x_24, 1); -lean_inc(x_30); -lean_inc(x_29); -lean_dec(x_24); -x_31 = l_Lean_Expr_const___override(x_5, x_6); -x_32 = l_Lean_mkApp7(x_31, x_7, x_8, x_9, x_10, x_21, x_18, x_29); -x_33 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_33, 0, x_32); -lean_ctor_set(x_33, 1, x_30); -return x_33; -} -} -else -{ -uint8_t x_34; -lean_dec(x_21); -lean_dec(x_18); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -x_34 = !lean_is_exclusive(x_24); -if (x_34 == 0) -{ -return x_24; -} -else -{ -lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_35 = lean_ctor_get(x_24, 0); -x_36 = lean_ctor_get(x_24, 1); -lean_inc(x_36); -lean_inc(x_35); -lean_dec(x_24); -x_37 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -return x_37; -} -} -} -else -{ -uint8_t x_38; -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_38 = !lean_is_exclusive(x_17); -if (x_38 == 0) -{ -return x_17; -} -else -{ -lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_39 = lean_ctor_get(x_17, 0); -x_40 = lean_ctor_get(x_17, 1); -lean_inc(x_40); -lean_inc(x_39); -lean_dec(x_17); -x_41 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_41, 0, x_39); -lean_ctor_set(x_41, 1, x_40); -return x_41; -} -} -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__1() { _start: { lean_object* x_1; @@ -234,7 +108,7 @@ x_1 = lean_mk_string_unchecked("Std", 3, 3); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__2() { _start: { lean_object* x_1; @@ -242,7 +116,7 @@ x_1 = lean_mk_string_unchecked("Tactic", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__3() { _start: { lean_object* x_1; @@ -250,1601 +124,1750 @@ x_1 = lean_mk_string_unchecked("BVDecide", 8, 8); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__4() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("BVPred", 6, 6); +x_1 = lean_mk_string_unchecked("Reflect", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__5() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("bin", 3, 3); +x_1 = lean_mk_string_unchecked("BitVec", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__6() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__6() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__2; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__4; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__5; -x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); -return x_6; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("ofBool_congr", 12, 12); +return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__7() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__7() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__6; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__3; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__4; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__5; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__6; +x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); +return x_7; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__8() { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("BVBinPred", 9, 9); -return x_1; +lean_object* x_11; lean_object* x_12; +x_11 = lean_ctor_get(x_1, 2); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_apply_6(x_11, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_12) == 0) +{ +uint8_t x_13; +x_13 = !lean_is_exclusive(x_12); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_14 = lean_ctor_get(x_12, 0); +x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__7; +x_16 = l_Lean_Expr_const___override(x_15, x_2); +x_17 = l_Lean_mkApp3(x_16, x_3, x_4, x_14); +lean_ctor_set(x_12, 0, x_17); +return x_12; +} +else +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_18 = lean_ctor_get(x_12, 0); +x_19 = lean_ctor_get(x_12, 1); +lean_inc(x_19); +lean_inc(x_18); +lean_dec(x_12); +x_20 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__7; +x_21 = l_Lean_Expr_const___override(x_20, x_2); +x_22 = l_Lean_mkApp3(x_21, x_3, x_4, x_18); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_19); +return x_23; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__9() { +else +{ +uint8_t x_24; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_24 = !lean_is_exclusive(x_12); +if (x_24 == 0) +{ +return x_12; +} +else +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_12, 0); +x_26 = lean_ctor_get(x_12, 1); +lean_inc(x_26); +lean_inc(x_25); +lean_dec(x_12); +x_27 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +return x_27; +} +} +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("eq", 2, 2); +x_1 = lean_mk_string_unchecked("ofBool", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__10() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__2() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__2; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__8; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__9; -x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); -return x_6; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__5; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__1; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__11() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__10; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__2; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__12() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__4() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("ult", 3, 3); +x_1 = lean_mk_string_unchecked("BVPred", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("getLsbD", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__13() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__2; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__8; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__12; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__3; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__4; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__5; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__14() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__13; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__6; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__8() { _start: { -lean_object* x_11; -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_1); -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of(x_1, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_11) == 0) +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(1u); +x_2 = l_Lean_mkNatLit(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__9() { +_start: { -lean_object* x_12; -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); -if (lean_obj_tag(x_12) == 0) +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(0u); +x_2 = l_Lean_mkNatLit(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: { -uint8_t x_13; -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -x_13 = !lean_is_exclusive(x_11); -if (x_13 == 0) +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_9 = lean_box(0); +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__3; +lean_inc(x_1); +x_11 = l_Lean_Expr_app___override(x_10, x_1); +x_12 = lean_unsigned_to_nat(1u); +x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom(x_11, x_12, x_3, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_13) == 0) { -lean_object* x_14; lean_object* x_15; -x_14 = lean_ctor_get(x_11, 0); -lean_dec(x_14); -x_15 = lean_box(0); -lean_ctor_set(x_11, 0, x_15); -return x_11; +uint8_t x_14; +x_14 = !lean_is_exclusive(x_13); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_15 = lean_ctor_get(x_13, 0); +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_15, 1); +lean_inc(x_17); +x_18 = lean_ctor_get(x_15, 3); +lean_inc(x_18); +x_19 = lean_unsigned_to_nat(0u); +lean_inc(x_16); +x_20 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_20, 0, x_16); +lean_ctor_set(x_20, 1, x_17); +lean_ctor_set(x_20, 2, x_19); +x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__7; +x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__8; +x_23 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__9; +lean_inc(x_18); +x_24 = l_Lean_mkApp3(x_21, x_22, x_18, x_23); +x_25 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_25, 0, x_16); +lean_closure_set(x_25, 1, x_18); +x_26 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1), 10, 3); +lean_closure_set(x_26, 0, x_15); +lean_closure_set(x_26, 1, x_9); +lean_closure_set(x_26, 2, x_1); +x_27 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_27, 0, x_25); +lean_closure_set(x_27, 1, x_26); +x_28 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_28, 0, x_20); +lean_ctor_set(x_28, 1, x_27); +lean_ctor_set(x_28, 2, x_24); +x_29 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_13, 0, x_29); +return x_13; } else { -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_11, 1); -lean_inc(x_16); -lean_dec(x_11); -x_17 = lean_box(0); -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_17); -lean_ctor_set(x_18, 1, x_16); -return x_18; +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_30 = lean_ctor_get(x_13, 0); +x_31 = lean_ctor_get(x_13, 1); +lean_inc(x_31); +lean_inc(x_30); +lean_dec(x_13); +x_32 = lean_ctor_get(x_30, 0); +lean_inc(x_32); +x_33 = lean_ctor_get(x_30, 1); +lean_inc(x_33); +x_34 = lean_ctor_get(x_30, 3); +lean_inc(x_34); +x_35 = lean_unsigned_to_nat(0u); +lean_inc(x_32); +x_36 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_36, 0, x_32); +lean_ctor_set(x_36, 1, x_33); +lean_ctor_set(x_36, 2, x_35); +x_37 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__7; +x_38 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__8; +x_39 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__9; +lean_inc(x_34); +x_40 = l_Lean_mkApp3(x_37, x_38, x_34, x_39); +x_41 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_41, 0, x_32); +lean_closure_set(x_41, 1, x_34); +x_42 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1), 10, 3); +lean_closure_set(x_42, 0, x_30); +lean_closure_set(x_42, 1, x_9); +lean_closure_set(x_42, 2, x_1); +x_43 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_43, 0, x_41); +lean_closure_set(x_43, 1, x_42); +x_44 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_44, 0, x_36); +lean_ctor_set(x_44, 1, x_43); +lean_ctor_set(x_44, 2, x_40); +x_45 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_45, 0, x_44); +x_46 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_46, 0, x_45); +lean_ctor_set(x_46, 1, x_31); +return x_46; } } else { -lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_19 = lean_ctor_get(x_11, 1); -lean_inc(x_19); -lean_dec(x_11); -x_20 = lean_ctor_get(x_12, 0); -lean_inc(x_20); -lean_dec(x_12); -lean_inc(x_2); -x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of(x_2, x_5, x_6, x_7, x_8, x_9, x_19); -if (lean_obj_tag(x_21) == 0) -{ -lean_object* x_22; -x_22 = lean_ctor_get(x_21, 0); -lean_inc(x_22); -if (lean_obj_tag(x_22) == 0) -{ -uint8_t x_23; -lean_dec(x_20); -lean_dec(x_4); -lean_dec(x_2); +uint8_t x_47; lean_dec(x_1); -x_23 = !lean_is_exclusive(x_21); -if (x_23 == 0) +x_47 = !lean_is_exclusive(x_13); +if (x_47 == 0) { -lean_object* x_24; lean_object* x_25; -x_24 = lean_ctor_get(x_21, 0); -lean_dec(x_24); -x_25 = lean_box(0); -lean_ctor_set(x_21, 0, x_25); -return x_21; +return x_13; } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_21, 1); -lean_inc(x_26); -lean_dec(x_21); -x_27 = lean_box(0); -x_28 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_28, 0, x_27); -lean_ctor_set(x_28, 1, x_26); -return x_28; +lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_48 = lean_ctor_get(x_13, 0); +x_49 = lean_ctor_get(x_13, 1); +lean_inc(x_49); +lean_inc(x_48); +lean_dec(x_13); +x_50 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_50, 0, x_48); +lean_ctor_set(x_50, 1, x_49); +return x_50; } } -else +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: { -uint8_t x_29; -x_29 = !lean_is_exclusive(x_21); -if (x_29 == 0) +lean_object* x_8; lean_object* x_9; +x_8 = lean_box(0); +x_9 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_9, 0, x_8); +lean_ctor_set(x_9, 1, x_7); +return x_9; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__1() { +_start: { -lean_object* x_30; uint8_t x_31; -x_30 = lean_ctor_get(x_21, 0); -lean_dec(x_30); -x_31 = !lean_is_exclusive(x_22); -if (x_31 == 0) +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__3___boxed), 7, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__2() { +_start: { -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; uint8_t x_38; -x_32 = lean_ctor_get(x_22, 0); -x_33 = lean_ctor_get(x_20, 0); -lean_inc(x_33); -x_34 = lean_ctor_get(x_20, 1); -lean_inc(x_34); -x_35 = lean_ctor_get(x_20, 2); -lean_inc(x_35); -x_36 = lean_ctor_get(x_20, 3); -lean_inc(x_36); -lean_dec(x_20); -x_37 = lean_ctor_get(x_32, 0); -lean_inc(x_37); -x_38 = lean_nat_dec_eq(x_33, x_37); -if (x_38 == 0) +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Bool", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__3() { +_start: { -lean_object* x_39; -lean_dec(x_37); -lean_dec(x_36); -lean_dec(x_35); -lean_dec(x_34); -lean_dec(x_33); -lean_free_object(x_22); -lean_dec(x_32); -lean_dec(x_4); -lean_dec(x_2); +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__2; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_1); +x_8 = lean_infer_type(x_1, x_3, x_4, x_5, x_6, x_7); +if (lean_obj_tag(x_8) == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_9 = lean_ctor_get(x_8, 0); +lean_inc(x_9); +x_10 = lean_ctor_get(x_8, 1); +lean_inc(x_10); +lean_dec(x_8); +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__1; +x_12 = l_Lean_Expr_cleanupAnnotations(x_9); +x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__3; +x_14 = l_Lean_Expr_isConstOf(x_12, x_13); +lean_dec(x_12); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; lean_dec(x_1); -x_39 = lean_box(0); -lean_ctor_set(x_21, 0, x_39); -return x_21; +x_15 = lean_box(0); +x_16 = lean_apply_7(x_11, x_15, x_2, x_3, x_4, x_5, x_6, x_10); +return x_16; } else { -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_40 = lean_ctor_get(x_32, 1); -lean_inc(x_40); -lean_inc(x_33); -x_41 = lean_alloc_ctor(0, 3, 1); -lean_ctor_set(x_41, 0, x_33); -lean_ctor_set(x_41, 1, x_34); -lean_ctor_set(x_41, 2, x_40); -lean_ctor_set_uint8(x_41, sizeof(void*)*3, x_3); -x_42 = lean_box(0); -lean_inc(x_33); -x_43 = l_Lean_mkNatLit(x_33); -x_44 = lean_ctor_get(x_32, 3); -lean_inc(x_44); -lean_inc(x_36); -x_45 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_45, 0, x_33); -lean_closure_set(x_45, 1, x_36); -lean_inc(x_43); -lean_inc(x_44); -x_46 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___lambda__1), 16, 9); -lean_closure_set(x_46, 0, x_35); -lean_closure_set(x_46, 1, x_37); -lean_closure_set(x_46, 2, x_44); -lean_closure_set(x_46, 3, x_32); -lean_closure_set(x_46, 4, x_4); -lean_closure_set(x_46, 5, x_42); -lean_closure_set(x_46, 6, x_43); -lean_closure_set(x_46, 7, x_1); -lean_closure_set(x_46, 8, x_2); -x_47 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_47, 0, x_45); -lean_closure_set(x_47, 1, x_46); -if (x_3 == 0) +lean_object* x_17; lean_object* x_18; +x_17 = lean_box(0); +x_18 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2(x_1, x_17, x_2, x_3, x_4, x_5, x_6, x_10); +return x_18; +} +} +else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_48 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__7; -x_49 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__11; -x_50 = l_Lean_mkApp4(x_48, x_43, x_36, x_49, x_44); -x_51 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_51, 0, x_41); -lean_ctor_set(x_51, 1, x_47); -lean_ctor_set(x_51, 2, x_50); -lean_ctor_set(x_22, 0, x_51); -return x_21; +uint8_t x_19; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_19 = !lean_is_exclusive(x_8); +if (x_19 == 0) +{ +return x_8; } else { -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_52 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__7; -x_53 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__14; -x_54 = l_Lean_mkApp4(x_52, x_43, x_36, x_53, x_44); -x_55 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_55, 0, x_41); -lean_ctor_set(x_55, 1, x_47); -lean_ctor_set(x_55, 2, x_54); -lean_ctor_set(x_22, 0, x_55); -return x_21; +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_8, 0); +x_21 = lean_ctor_get(x_8, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_8); +x_22 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_22, 0, x_20); +lean_ctor_set(x_22, 1, x_21); +return x_22; } } } -else +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: { -lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; -x_56 = lean_ctor_get(x_22, 0); -lean_inc(x_56); -lean_dec(x_22); -x_57 = lean_ctor_get(x_20, 0); -lean_inc(x_57); -x_58 = lean_ctor_get(x_20, 1); -lean_inc(x_58); -x_59 = lean_ctor_get(x_20, 2); -lean_inc(x_59); -x_60 = lean_ctor_get(x_20, 3); -lean_inc(x_60); -lean_dec(x_20); -x_61 = lean_ctor_get(x_56, 0); -lean_inc(x_61); -x_62 = lean_nat_dec_eq(x_57, x_61); -if (x_62 == 0) +lean_object* x_9; +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_2); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: { -lean_object* x_63; -lean_dec(x_61); -lean_dec(x_60); -lean_dec(x_59); -lean_dec(x_58); -lean_dec(x_57); -lean_dec(x_56); +lean_object* x_8; +x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_63 = lean_box(0); -lean_ctor_set(x_21, 0, x_63); -return x_21; +return x_8; } -else +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +_start: { -lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; -x_64 = lean_ctor_get(x_56, 1); -lean_inc(x_64); -lean_inc(x_57); -x_65 = lean_alloc_ctor(0, 3, 1); -lean_ctor_set(x_65, 0, x_57); -lean_ctor_set(x_65, 1, x_58); -lean_ctor_set(x_65, 2, x_64); -lean_ctor_set_uint8(x_65, sizeof(void*)*3, x_3); -x_66 = lean_box(0); -lean_inc(x_57); -x_67 = l_Lean_mkNatLit(x_57); -x_68 = lean_ctor_get(x_56, 3); -lean_inc(x_68); -lean_inc(x_60); -x_69 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_69, 0, x_57); -lean_closure_set(x_69, 1, x_60); -lean_inc(x_67); -lean_inc(x_68); -x_70 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___lambda__1), 16, 9); -lean_closure_set(x_70, 0, x_59); -lean_closure_set(x_70, 1, x_61); -lean_closure_set(x_70, 2, x_68); -lean_closure_set(x_70, 3, x_56); -lean_closure_set(x_70, 4, x_4); -lean_closure_set(x_70, 5, x_66); -lean_closure_set(x_70, 6, x_67); -lean_closure_set(x_70, 7, x_1); -lean_closure_set(x_70, 8, x_2); -x_71 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_71, 0, x_69); -lean_closure_set(x_71, 1, x_70); -if (x_3 == 0) +lean_object* x_17; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +x_17 = lean_apply_6(x_1, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_17) == 0) { -lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; -x_72 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__7; -x_73 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__11; -x_74 = l_Lean_mkApp4(x_72, x_67, x_60, x_73, x_68); -x_75 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_75, 0, x_65); -lean_ctor_set(x_75, 1, x_71); -lean_ctor_set(x_75, 2, x_74); -x_76 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_76, 0, x_75); -lean_ctor_set(x_21, 0, x_76); -return x_21; +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); +lean_dec(x_17); +x_20 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr(x_2, x_3, x_11, x_12, x_13, x_14, x_15, x_19); +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +x_23 = lean_ctor_get(x_4, 2); +lean_inc(x_23); +lean_dec(x_4); +x_24 = lean_apply_6(x_23, x_11, x_12, x_13, x_14, x_15, x_22); +if (lean_obj_tag(x_24) == 0) +{ +uint8_t x_25; +x_25 = !lean_is_exclusive(x_24); +if (x_25 == 0) +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_24, 0); +x_27 = l_Lean_Expr_const___override(x_5, x_6); +x_28 = l_Lean_mkApp7(x_27, x_7, x_8, x_9, x_10, x_21, x_18, x_26); +lean_ctor_set(x_24, 0, x_28); +return x_24; } else { -lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; -x_77 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__7; -x_78 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__14; -x_79 = l_Lean_mkApp4(x_77, x_67, x_60, x_78, x_68); -x_80 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_80, 0, x_65); -lean_ctor_set(x_80, 1, x_71); -lean_ctor_set(x_80, 2, x_79); -x_81 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_81, 0, x_80); -lean_ctor_set(x_21, 0, x_81); -return x_21; -} -} +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_29 = lean_ctor_get(x_24, 0); +x_30 = lean_ctor_get(x_24, 1); +lean_inc(x_30); +lean_inc(x_29); +lean_dec(x_24); +x_31 = l_Lean_Expr_const___override(x_5, x_6); +x_32 = l_Lean_mkApp7(x_31, x_7, x_8, x_9, x_10, x_21, x_18, x_29); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_30); +return x_33; } } else { -lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; uint8_t x_90; -x_82 = lean_ctor_get(x_21, 1); -lean_inc(x_82); +uint8_t x_34; lean_dec(x_21); -x_83 = lean_ctor_get(x_22, 0); -lean_inc(x_83); -if (lean_is_exclusive(x_22)) { - lean_ctor_release(x_22, 0); - x_84 = x_22; -} else { - lean_dec_ref(x_22); - x_84 = lean_box(0); +lean_dec(x_18); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_34 = !lean_is_exclusive(x_24); +if (x_34 == 0) +{ +return x_24; } -x_85 = lean_ctor_get(x_20, 0); -lean_inc(x_85); -x_86 = lean_ctor_get(x_20, 1); -lean_inc(x_86); -x_87 = lean_ctor_get(x_20, 2); -lean_inc(x_87); -x_88 = lean_ctor_get(x_20, 3); -lean_inc(x_88); -lean_dec(x_20); -x_89 = lean_ctor_get(x_83, 0); -lean_inc(x_89); -x_90 = lean_nat_dec_eq(x_85, x_89); -if (x_90 == 0) +else { -lean_object* x_91; lean_object* x_92; -lean_dec(x_89); -lean_dec(x_88); -lean_dec(x_87); -lean_dec(x_86); -lean_dec(x_85); -lean_dec(x_84); -lean_dec(x_83); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -x_91 = lean_box(0); -x_92 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_92, 0, x_91); -lean_ctor_set(x_92, 1, x_82); -return x_92; -} -else -{ -lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; -x_93 = lean_ctor_get(x_83, 1); -lean_inc(x_93); -lean_inc(x_85); -x_94 = lean_alloc_ctor(0, 3, 1); -lean_ctor_set(x_94, 0, x_85); -lean_ctor_set(x_94, 1, x_86); -lean_ctor_set(x_94, 2, x_93); -lean_ctor_set_uint8(x_94, sizeof(void*)*3, x_3); -x_95 = lean_box(0); -lean_inc(x_85); -x_96 = l_Lean_mkNatLit(x_85); -x_97 = lean_ctor_get(x_83, 3); -lean_inc(x_97); -lean_inc(x_88); -x_98 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_98, 0, x_85); -lean_closure_set(x_98, 1, x_88); -lean_inc(x_96); -lean_inc(x_97); -x_99 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___lambda__1), 16, 9); -lean_closure_set(x_99, 0, x_87); -lean_closure_set(x_99, 1, x_89); -lean_closure_set(x_99, 2, x_97); -lean_closure_set(x_99, 3, x_83); -lean_closure_set(x_99, 4, x_4); -lean_closure_set(x_99, 5, x_95); -lean_closure_set(x_99, 6, x_96); -lean_closure_set(x_99, 7, x_1); -lean_closure_set(x_99, 8, x_2); -x_100 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_100, 0, x_98); -lean_closure_set(x_100, 1, x_99); -if (x_3 == 0) -{ -lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; -x_101 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__7; -x_102 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__11; -x_103 = l_Lean_mkApp4(x_101, x_96, x_88, x_102, x_97); -x_104 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_104, 0, x_94); -lean_ctor_set(x_104, 1, x_100); -lean_ctor_set(x_104, 2, x_103); -if (lean_is_scalar(x_84)) { - x_105 = lean_alloc_ctor(1, 1, 0); -} else { - x_105 = x_84; -} -lean_ctor_set(x_105, 0, x_104); -x_106 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_106, 0, x_105); -lean_ctor_set(x_106, 1, x_82); -return x_106; -} -else -{ -lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; -x_107 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__7; -x_108 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__14; -x_109 = l_Lean_mkApp4(x_107, x_96, x_88, x_108, x_97); -x_110 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_110, 0, x_94); -lean_ctor_set(x_110, 1, x_100); -lean_ctor_set(x_110, 2, x_109); -if (lean_is_scalar(x_84)) { - x_111 = lean_alloc_ctor(1, 1, 0); -} else { - x_111 = x_84; -} -lean_ctor_set(x_111, 0, x_110); -x_112 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_112, 0, x_111); -lean_ctor_set(x_112, 1, x_82); -return x_112; -} -} -} -} -} -else -{ -uint8_t x_113; -lean_dec(x_20); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -x_113 = !lean_is_exclusive(x_21); -if (x_113 == 0) -{ -return x_21; -} -else -{ -lean_object* x_114; lean_object* x_115; lean_object* x_116; -x_114 = lean_ctor_get(x_21, 0); -x_115 = lean_ctor_get(x_21, 1); -lean_inc(x_115); -lean_inc(x_114); -lean_dec(x_21); -x_116 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_116, 0, x_114); -lean_ctor_set(x_116, 1, x_115); -return x_116; -} +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_24, 0); +x_36 = lean_ctor_get(x_24, 1); +lean_inc(x_36); +lean_inc(x_35); +lean_dec(x_24); +x_37 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +return x_37; } } } else { -uint8_t x_117; +uint8_t x_38; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_117 = !lean_is_exclusive(x_11); -if (x_117 == 0) +x_38 = !lean_is_exclusive(x_17); +if (x_38 == 0) { -return x_11; +return x_17; } else { -lean_object* x_118; lean_object* x_119; lean_object* x_120; -x_118 = lean_ctor_get(x_11, 0); -x_119 = lean_ctor_get(x_11, 1); -lean_inc(x_119); -lean_inc(x_118); -lean_dec(x_11); -x_120 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_120, 0, x_118); -lean_ctor_set(x_120, 1, x_119); -return x_120; +lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = lean_ctor_get(x_17, 0); +x_40 = lean_ctor_get(x_17, 1); +lean_inc(x_40); +lean_inc(x_39); +lean_dec(x_17); +x_41 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_41, 0, x_39); +lean_ctor_set(x_41, 1, x_40); +return x_41; } } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__1() { _start: { -uint8_t x_11; lean_object* x_12; -x_11 = lean_unbox(x_3); -lean_dec(x_3); -x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection(x_1, x_2, x_11, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_12; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("bin", 3, 3); +return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Reflect", 7, 7); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__3; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__4; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__1; +x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); +return x_6; +} } +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__2; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__2() { +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__4() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("BitVec", 6, 6); +x_1 = lean_mk_string_unchecked("BVBinPred", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__5() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("getLsbD_congr", 13, 13); +x_1 = lean_mk_string_unchecked("eq", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__6() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__2; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__2; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__3; -x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); -return x_7; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__3; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__4; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__5; +x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); +return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__7() { _start: { -lean_object* x_13; lean_object* x_14; -x_13 = lean_ctor_get(x_1, 2); -lean_inc(x_13); -lean_dec(x_1); -x_14 = lean_apply_6(x_13, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_14) == 0) -{ -uint8_t x_15; -x_15 = !lean_is_exclusive(x_14); -if (x_15 == 0) +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__6; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__8() { +_start: { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_16 = lean_ctor_get(x_14, 0); -x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__4; -x_18 = l_Lean_Expr_const___override(x_17, x_2); -x_19 = l_Lean_mkApp5(x_18, x_3, x_4, x_5, x_6, x_16); -lean_ctor_set(x_14, 0, x_19); -return x_14; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("ult", 3, 3); +return x_1; } -else +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__9() { +_start: { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_20 = lean_ctor_get(x_14, 0); -x_21 = lean_ctor_get(x_14, 1); -lean_inc(x_21); -lean_inc(x_20); -lean_dec(x_14); -x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__4; -x_23 = l_Lean_Expr_const___override(x_22, x_2); -x_24 = l_Lean_mkApp5(x_23, x_3, x_4, x_5, x_6, x_20); -x_25 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_25, 0, x_24); -lean_ctor_set(x_25, 1, x_21); -return x_25; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__3; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__4; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__8; +x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); +return x_6; } } -else -{ -uint8_t x_26; -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_26 = !lean_is_exclusive(x_14); -if (x_26 == 0) -{ -return x_14; -} -else -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_14, 0); -x_28 = lean_ctor_get(x_14, 1); -lean_inc(x_28); -lean_inc(x_27); -lean_dec(x_14); -x_29 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_29, 0, x_27); -lean_ctor_set(x_29, 1, x_28); -return x_29; -} -} -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("getLsbD", 7, 7); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__2; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__4; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__1; -x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); -return x_6; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__3() { -_start: +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__10() { +_start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__2; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__9; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_9; +lean_object* x_11; +lean_inc(x_9); +lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -lean_inc(x_4); lean_inc(x_1); -x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of(x_1, x_3, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_9) == 0) +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(x_1, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_11) == 0) { -lean_object* x_10; -x_10 = lean_ctor_get(x_9, 0); -lean_inc(x_10); -if (lean_obj_tag(x_10) == 0) +lean_object* x_12; +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +if (lean_obj_tag(x_12) == 0) { -uint8_t x_11; +uint8_t x_13; +lean_dec(x_9); +lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_11 = !lean_is_exclusive(x_9); -if (x_11 == 0) +x_13 = !lean_is_exclusive(x_11); +if (x_13 == 0) { -lean_object* x_12; lean_object* x_13; -x_12 = lean_ctor_get(x_9, 0); -lean_dec(x_12); -x_13 = lean_box(0); -lean_ctor_set(x_9, 0, x_13); -return x_9; +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_11, 0); +lean_dec(x_14); +x_15 = lean_box(0); +lean_ctor_set(x_11, 0, x_15); +return x_11; } else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_14 = lean_ctor_get(x_9, 1); -lean_inc(x_14); -lean_dec(x_9); -x_15 = lean_box(0); -x_16 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_16, 0, x_15); -lean_ctor_set(x_16, 1, x_14); -return x_16; +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_11, 1); +lean_inc(x_16); +lean_dec(x_11); +x_17 = lean_box(0); +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set(x_18, 1, x_16); +return x_18; } } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_9, 1); -lean_inc(x_17); -lean_dec(x_9); -x_18 = lean_ctor_get(x_10, 0); -lean_inc(x_18); -lean_dec(x_10); -x_19 = l_Lean_Meta_getNatValue_x3f(x_2, x_4, x_5, x_6, x_7, x_17); -if (lean_obj_tag(x_19) == 0) -{ -lean_object* x_20; -x_20 = lean_ctor_get(x_19, 0); +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_11, 1); +lean_inc(x_19); +lean_dec(x_11); +x_20 = lean_ctor_get(x_12, 0); lean_inc(x_20); -if (lean_obj_tag(x_20) == 0) +lean_dec(x_12); +lean_inc(x_2); +x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(x_2, x_5, x_6, x_7, x_8, x_9, x_19); +if (lean_obj_tag(x_21) == 0) { -uint8_t x_21; -lean_dec(x_18); +lean_object* x_22; +x_22 = lean_ctor_get(x_21, 0); +lean_inc(x_22); +if (lean_obj_tag(x_22) == 0) +{ +uint8_t x_23; +lean_dec(x_20); +lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_21 = !lean_is_exclusive(x_19); -if (x_21 == 0) +x_23 = !lean_is_exclusive(x_21); +if (x_23 == 0) { -lean_object* x_22; lean_object* x_23; -x_22 = lean_ctor_get(x_19, 0); -lean_dec(x_22); -x_23 = lean_box(0); -lean_ctor_set(x_19, 0, x_23); -return x_19; +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_21, 0); +lean_dec(x_24); +x_25 = lean_box(0); +lean_ctor_set(x_21, 0, x_25); +return x_21; } else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_19, 1); -lean_inc(x_24); -lean_dec(x_19); -x_25 = lean_box(0); -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_26, 1, x_24); -return x_26; +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_21, 1); +lean_inc(x_26); +lean_dec(x_21); +x_27 = lean_box(0); +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_26); +return x_28; } } else { -uint8_t x_27; -x_27 = !lean_is_exclusive(x_19); -if (x_27 == 0) -{ -lean_object* x_28; uint8_t x_29; -x_28 = lean_ctor_get(x_19, 0); -lean_dec(x_28); -x_29 = !lean_is_exclusive(x_20); +uint8_t x_29; +x_29 = !lean_is_exclusive(x_21); if (x_29 == 0) { -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_30 = lean_ctor_get(x_20, 0); -x_31 = lean_ctor_get(x_18, 0); -lean_inc(x_31); -x_32 = lean_ctor_get(x_18, 1); -lean_inc(x_32); -x_33 = lean_ctor_get(x_18, 3); -lean_inc(x_33); -lean_inc(x_31); -x_34 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_34, 0, x_31); -lean_ctor_set(x_34, 1, x_32); -lean_ctor_set(x_34, 2, x_30); -x_35 = lean_box(0); -lean_inc(x_31); -x_36 = l_Lean_mkNatLit(x_31); -x_37 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__3; -lean_inc(x_2); +lean_object* x_30; uint8_t x_31; +x_30 = lean_ctor_get(x_21, 0); +lean_dec(x_30); +x_31 = !lean_is_exclusive(x_22); +if (x_31 == 0) +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; uint8_t x_38; +x_32 = lean_ctor_get(x_22, 0); +x_33 = lean_ctor_get(x_20, 0); lean_inc(x_33); +x_34 = lean_ctor_get(x_20, 1); +lean_inc(x_34); +x_35 = lean_ctor_get(x_20, 2); +lean_inc(x_35); +x_36 = lean_ctor_get(x_20, 3); lean_inc(x_36); -x_38 = l_Lean_mkApp3(x_37, x_36, x_33, x_2); -x_39 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_39, 0, x_31); -lean_closure_set(x_39, 1, x_33); -x_40 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1), 12, 5); -lean_closure_set(x_40, 0, x_18); -lean_closure_set(x_40, 1, x_35); -lean_closure_set(x_40, 2, x_2); -lean_closure_set(x_40, 3, x_36); -lean_closure_set(x_40, 4, x_1); -x_41 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_41, 0, x_39); -lean_closure_set(x_41, 1, x_40); -x_42 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_42, 0, x_34); -lean_ctor_set(x_42, 1, x_41); -lean_ctor_set(x_42, 2, x_38); -lean_ctor_set(x_20, 0, x_42); -return x_19; +lean_dec(x_20); +x_37 = lean_ctor_get(x_32, 0); +lean_inc(x_37); +x_38 = lean_nat_dec_eq(x_33, x_37); +if (x_38 == 0) +{ +lean_object* x_39; +lean_dec(x_37); +lean_dec(x_36); +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_33); +lean_free_object(x_22); +lean_dec(x_32); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_39 = lean_box(0); +lean_ctor_set(x_21, 0, x_39); +return x_21; } else { -lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; -x_43 = lean_ctor_get(x_20, 0); -lean_inc(x_43); -lean_dec(x_20); -x_44 = lean_ctor_get(x_18, 0); -lean_inc(x_44); -x_45 = lean_ctor_get(x_18, 1); -lean_inc(x_45); -x_46 = lean_ctor_get(x_18, 3); -lean_inc(x_46); -lean_inc(x_44); -x_47 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_47, 0, x_44); -lean_ctor_set(x_47, 1, x_45); -lean_ctor_set(x_47, 2, x_43); -x_48 = lean_box(0); +lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_40 = lean_ctor_get(x_32, 1); +lean_inc(x_40); +lean_inc(x_33); +x_41 = lean_alloc_ctor(0, 3, 1); +lean_ctor_set(x_41, 0, x_33); +lean_ctor_set(x_41, 1, x_34); +lean_ctor_set(x_41, 2, x_40); +lean_ctor_set_uint8(x_41, sizeof(void*)*3, x_3); +x_42 = lean_box(0); +lean_inc(x_33); +x_43 = l_Lean_mkNatLit(x_33); +x_44 = lean_ctor_get(x_32, 3); lean_inc(x_44); -x_49 = l_Lean_mkNatLit(x_44); -x_50 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__3; -lean_inc(x_2); -lean_inc(x_46); -lean_inc(x_49); -x_51 = l_Lean_mkApp3(x_50, x_49, x_46, x_2); -x_52 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_52, 0, x_44); -lean_closure_set(x_52, 1, x_46); -x_53 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1), 12, 5); -lean_closure_set(x_53, 0, x_18); -lean_closure_set(x_53, 1, x_48); -lean_closure_set(x_53, 2, x_2); -lean_closure_set(x_53, 3, x_49); -lean_closure_set(x_53, 4, x_1); -x_54 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_54, 0, x_52); -lean_closure_set(x_54, 1, x_53); +lean_inc(x_36); +x_45 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_45, 0, x_33); +lean_closure_set(x_45, 1, x_36); +lean_inc(x_43); +lean_inc(x_44); +x_46 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___lambda__1), 16, 9); +lean_closure_set(x_46, 0, x_35); +lean_closure_set(x_46, 1, x_37); +lean_closure_set(x_46, 2, x_44); +lean_closure_set(x_46, 3, x_32); +lean_closure_set(x_46, 4, x_4); +lean_closure_set(x_46, 5, x_42); +lean_closure_set(x_46, 6, x_43); +lean_closure_set(x_46, 7, x_1); +lean_closure_set(x_46, 8, x_2); +x_47 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_47, 0, x_45); +lean_closure_set(x_47, 1, x_46); +if (x_3 == 0) +{ +lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_48 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__3; +x_49 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__7; +x_50 = l_Lean_mkApp4(x_48, x_43, x_36, x_49, x_44); +x_51 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_51, 0, x_41); +lean_ctor_set(x_51, 1, x_47); +lean_ctor_set(x_51, 2, x_50); +lean_ctor_set(x_22, 0, x_51); +return x_21; +} +else +{ +lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; +x_52 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__3; +x_53 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__10; +x_54 = l_Lean_mkApp4(x_52, x_43, x_36, x_53, x_44); x_55 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_55, 0, x_47); -lean_ctor_set(x_55, 1, x_54); -lean_ctor_set(x_55, 2, x_51); -x_56 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_56, 0, x_55); -lean_ctor_set(x_19, 0, x_56); -return x_19; +lean_ctor_set(x_55, 0, x_41); +lean_ctor_set(x_55, 1, x_47); +lean_ctor_set(x_55, 2, x_54); +lean_ctor_set(x_22, 0, x_55); +return x_21; +} } } else { -lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_57 = lean_ctor_get(x_19, 1); +lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; +x_56 = lean_ctor_get(x_22, 0); +lean_inc(x_56); +lean_dec(x_22); +x_57 = lean_ctor_get(x_20, 0); lean_inc(x_57); -lean_dec(x_19); -x_58 = lean_ctor_get(x_20, 0); +x_58 = lean_ctor_get(x_20, 1); lean_inc(x_58); -if (lean_is_exclusive(x_20)) { - lean_ctor_release(x_20, 0); - x_59 = x_20; -} else { - lean_dec_ref(x_20); - x_59 = lean_box(0); -} -x_60 = lean_ctor_get(x_18, 0); +x_59 = lean_ctor_get(x_20, 2); +lean_inc(x_59); +x_60 = lean_ctor_get(x_20, 3); lean_inc(x_60); -x_61 = lean_ctor_get(x_18, 1); +lean_dec(x_20); +x_61 = lean_ctor_get(x_56, 0); lean_inc(x_61); -x_62 = lean_ctor_get(x_18, 3); -lean_inc(x_62); -lean_inc(x_60); -x_63 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_63, 0, x_60); -lean_ctor_set(x_63, 1, x_61); -lean_ctor_set(x_63, 2, x_58); -x_64 = lean_box(0); -lean_inc(x_60); -x_65 = l_Lean_mkNatLit(x_60); -x_66 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__3; -lean_inc(x_2); -lean_inc(x_62); -lean_inc(x_65); -x_67 = l_Lean_mkApp3(x_66, x_65, x_62, x_2); -x_68 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_68, 0, x_60); -lean_closure_set(x_68, 1, x_62); -x_69 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1), 12, 5); -lean_closure_set(x_69, 0, x_18); -lean_closure_set(x_69, 1, x_64); -lean_closure_set(x_69, 2, x_2); -lean_closure_set(x_69, 3, x_65); -lean_closure_set(x_69, 4, x_1); -x_70 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_70, 0, x_68); -lean_closure_set(x_70, 1, x_69); -x_71 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_71, 0, x_63); -lean_ctor_set(x_71, 1, x_70); -lean_ctor_set(x_71, 2, x_67); -if (lean_is_scalar(x_59)) { - x_72 = lean_alloc_ctor(1, 1, 0); -} else { - x_72 = x_59; -} -lean_ctor_set(x_72, 0, x_71); -x_73 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_73, 0, x_72); -lean_ctor_set(x_73, 1, x_57); -return x_73; -} -} -} -else +x_62 = lean_nat_dec_eq(x_57, x_61); +if (x_62 == 0) { -uint8_t x_74; -lean_dec(x_18); +lean_object* x_63; +lean_dec(x_61); +lean_dec(x_60); +lean_dec(x_59); +lean_dec(x_58); +lean_dec(x_57); +lean_dec(x_56); +lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_74 = !lean_is_exclusive(x_19); -if (x_74 == 0) -{ -return x_19; -} -else -{ -lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_75 = lean_ctor_get(x_19, 0); -x_76 = lean_ctor_get(x_19, 1); -lean_inc(x_76); -lean_inc(x_75); -lean_dec(x_19); -x_77 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_77, 0, x_75); -lean_ctor_set(x_77, 1, x_76); -return x_77; -} -} -} +x_63 = lean_box(0); +lean_ctor_set(x_21, 0, x_63); +return x_21; } else { -uint8_t x_78; -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -x_78 = !lean_is_exclusive(x_9); -if (x_78 == 0) +lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; +x_64 = lean_ctor_get(x_56, 1); +lean_inc(x_64); +lean_inc(x_57); +x_65 = lean_alloc_ctor(0, 3, 1); +lean_ctor_set(x_65, 0, x_57); +lean_ctor_set(x_65, 1, x_58); +lean_ctor_set(x_65, 2, x_64); +lean_ctor_set_uint8(x_65, sizeof(void*)*3, x_3); +x_66 = lean_box(0); +lean_inc(x_57); +x_67 = l_Lean_mkNatLit(x_57); +x_68 = lean_ctor_get(x_56, 3); +lean_inc(x_68); +lean_inc(x_60); +x_69 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_69, 0, x_57); +lean_closure_set(x_69, 1, x_60); +lean_inc(x_67); +lean_inc(x_68); +x_70 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___lambda__1), 16, 9); +lean_closure_set(x_70, 0, x_59); +lean_closure_set(x_70, 1, x_61); +lean_closure_set(x_70, 2, x_68); +lean_closure_set(x_70, 3, x_56); +lean_closure_set(x_70, 4, x_4); +lean_closure_set(x_70, 5, x_66); +lean_closure_set(x_70, 6, x_67); +lean_closure_set(x_70, 7, x_1); +lean_closure_set(x_70, 8, x_2); +x_71 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_71, 0, x_69); +lean_closure_set(x_71, 1, x_70); +if (x_3 == 0) { -return x_9; +lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; +x_72 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__3; +x_73 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__7; +x_74 = l_Lean_mkApp4(x_72, x_67, x_60, x_73, x_68); +x_75 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_75, 0, x_65); +lean_ctor_set(x_75, 1, x_71); +lean_ctor_set(x_75, 2, x_74); +x_76 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_76, 0, x_75); +lean_ctor_set(x_21, 0, x_76); +return x_21; } else { -lean_object* x_79; lean_object* x_80; lean_object* x_81; -x_79 = lean_ctor_get(x_9, 0); -x_80 = lean_ctor_get(x_9, 1); -lean_inc(x_80); -lean_inc(x_79); -lean_dec(x_9); -x_81 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_81, 0, x_79); -lean_ctor_set(x_81, 1, x_80); -return x_81; +lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_77 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__3; +x_78 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__10; +x_79 = l_Lean_mkApp4(x_77, x_67, x_60, x_78, x_68); +x_80 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_80, 0, x_65); +lean_ctor_set(x_80, 1, x_71); +lean_ctor_set(x_80, 2, x_79); +x_81 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_81, 0, x_80); +lean_ctor_set(x_21, 0, x_81); +return x_21; } } } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__3___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("ult_congr", 9, 9); -return x_1; -} +lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; uint8_t x_90; +x_82 = lean_ctor_get(x_21, 1); +lean_inc(x_82); +lean_dec(x_21); +x_83 = lean_ctor_get(x_22, 0); +lean_inc(x_83); +if (lean_is_exclusive(x_22)) { + lean_ctor_release(x_22, 0); + x_84 = x_22; +} else { + lean_dec_ref(x_22); + x_84 = lean_box(0); } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__3___closed__2() { -_start: +x_85 = lean_ctor_get(x_20, 0); +lean_inc(x_85); +x_86 = lean_ctor_get(x_20, 1); +lean_inc(x_86); +x_87 = lean_ctor_get(x_20, 2); +lean_inc(x_87); +x_88 = lean_ctor_get(x_20, 3); +lean_inc(x_88); +lean_dec(x_20); +x_89 = lean_ctor_get(x_83, 0); +lean_inc(x_89); +x_90 = lean_nat_dec_eq(x_85, x_89); +if (x_90 == 0) { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__2; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__2; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__3___closed__1; -x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); -return x_7; -} +lean_object* x_91; lean_object* x_92; +lean_dec(x_89); +lean_dec(x_88); +lean_dec(x_87); +lean_dec(x_86); +lean_dec(x_85); +lean_dec(x_84); +lean_dec(x_83); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_91 = lean_box(0); +x_92 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_92, 0, x_91); +lean_ctor_set(x_92, 1, x_82); +return x_92; } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: +else { -uint8_t x_9; lean_object* x_10; lean_object* x_11; -x_9 = 1; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__3___closed__2; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection(x_1, x_2, x_9, x_10, x_3, x_4, x_5, x_6, x_7, x_8); -return x_11; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__4___closed__1() { -_start: +lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; +x_93 = lean_ctor_get(x_83, 1); +lean_inc(x_93); +lean_inc(x_85); +x_94 = lean_alloc_ctor(0, 3, 1); +lean_ctor_set(x_94, 0, x_85); +lean_ctor_set(x_94, 1, x_86); +lean_ctor_set(x_94, 2, x_93); +lean_ctor_set_uint8(x_94, sizeof(void*)*3, x_3); +x_95 = lean_box(0); +lean_inc(x_85); +x_96 = l_Lean_mkNatLit(x_85); +x_97 = lean_ctor_get(x_83, 3); +lean_inc(x_97); +lean_inc(x_88); +x_98 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_98, 0, x_85); +lean_closure_set(x_98, 1, x_88); +lean_inc(x_96); +lean_inc(x_97); +x_99 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___lambda__1), 16, 9); +lean_closure_set(x_99, 0, x_87); +lean_closure_set(x_99, 1, x_89); +lean_closure_set(x_99, 2, x_97); +lean_closure_set(x_99, 3, x_83); +lean_closure_set(x_99, 4, x_4); +lean_closure_set(x_99, 5, x_95); +lean_closure_set(x_99, 6, x_96); +lean_closure_set(x_99, 7, x_1); +lean_closure_set(x_99, 8, x_2); +x_100 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_100, 0, x_98); +lean_closure_set(x_100, 1, x_99); +if (x_3 == 0) { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("beq_congr", 9, 9); -return x_1; +lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; +x_101 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__3; +x_102 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__7; +x_103 = l_Lean_mkApp4(x_101, x_96, x_88, x_102, x_97); +x_104 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_104, 0, x_94); +lean_ctor_set(x_104, 1, x_100); +lean_ctor_set(x_104, 2, x_103); +if (lean_is_scalar(x_84)) { + x_105 = lean_alloc_ctor(1, 1, 0); +} else { + x_105 = x_84; } +lean_ctor_set(x_105, 0, x_104); +x_106 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_106, 0, x_105); +lean_ctor_set(x_106, 1, x_82); +return x_106; } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__4___closed__2() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__2; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__2; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__4___closed__1; -x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); -return x_7; +lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; +x_107 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__3; +x_108 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__10; +x_109 = l_Lean_mkApp4(x_107, x_96, x_88, x_108, x_97); +x_110 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_110, 0, x_94); +lean_ctor_set(x_110, 1, x_100); +lean_ctor_set(x_110, 2, x_109); +if (lean_is_scalar(x_84)) { + x_111 = lean_alloc_ctor(1, 1, 0); +} else { + x_111 = x_84; } +lean_ctor_set(x_111, 0, x_110); +x_112 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_112, 0, x_111); +lean_ctor_set(x_112, 1, x_82); +return x_112; } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -uint8_t x_10; lean_object* x_11; lean_object* x_12; -x_10 = 0; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__4___closed__2; -x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection(x_1, x_2, x_10, x_11, x_4, x_5, x_6, x_7, x_8, x_9); -return x_12; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; lean_object* x_9; -x_8 = lean_box(0); -x_9 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_9, 0, x_8); -lean_ctor_set(x_9, 1, x_7); -return x_9; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__6___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__5___boxed), 7, 0); -return x_1; -} +uint8_t x_113; +lean_dec(x_20); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_113 = !lean_is_exclusive(x_21); +if (x_113 == 0) +{ +return x_21; } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__6___closed__2() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__2; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_114; lean_object* x_115; lean_object* x_116; +x_114 = lean_ctor_get(x_21, 0); +x_115 = lean_ctor_get(x_21, 1); +lean_inc(x_115); +lean_inc(x_114); +lean_dec(x_21); +x_116 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_116, 0, x_114); +lean_ctor_set(x_116, 1, x_115); +return x_116; +} } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__6___closed__1; -x_11 = l_Lean_Expr_cleanupAnnotations(x_1); -x_12 = l_Lean_Expr_isApp(x_11); -if (x_12 == 0) -{ -lean_object* x_13; lean_object* x_14; -lean_dec(x_11); -lean_dec(x_3); -lean_dec(x_2); -x_13 = lean_box(0); -x_14 = lean_apply_7(x_10, x_13, x_4, x_5, x_6, x_7, x_8, x_9); -return x_14; } else { -lean_object* x_15; lean_object* x_16; uint8_t x_17; -x_15 = l_Lean_Expr_appFnCleanup(x_11, lean_box(0)); -x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__6___closed__2; -x_17 = l_Lean_Expr_isConstOf(x_15, x_16); -lean_dec(x_15); -if (x_17 == 0) -{ -lean_object* x_18; lean_object* x_19; -lean_dec(x_3); +uint8_t x_117; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); lean_dec(x_2); -x_18 = lean_box(0); -x_19 = lean_apply_7(x_10, x_18, x_4, x_5, x_6, x_7, x_8, x_9); -return x_19; +lean_dec(x_1); +x_117 = !lean_is_exclusive(x_11); +if (x_117 == 0) +{ +return x_11; } else { -lean_object* x_20; lean_object* x_21; -x_20 = lean_box(0); -x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__4(x_2, x_3, x_20, x_4, x_5, x_6, x_7, x_8, x_9); -return x_21; +lean_object* x_118; lean_object* x_119; lean_object* x_120; +x_118 = lean_ctor_get(x_11, 0); +x_119 = lean_ctor_get(x_11, 1); +lean_inc(x_119); +lean_inc(x_118); +lean_dec(x_11); +x_120 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_120, 0, x_118); +lean_ctor_set(x_120, 1, x_119); +return x_120; +} +} } } +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +uint8_t x_11; lean_object* x_12; +x_11 = lean_unbox(x_3); +lean_dec(x_3); +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection(x_1, x_2, x_11, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_12; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__7___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__1___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("ofBool_congr", 12, 12); +x_1 = lean_mk_string_unchecked("getLsbD_congr", 13, 13); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__7___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__2; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__2; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__7___closed__1; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__3; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__4; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__5; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__1___closed__1; x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_11; lean_object* x_12; -x_11 = lean_ctor_get(x_1, 2); -lean_inc(x_11); +lean_object* x_13; lean_object* x_14; +x_13 = lean_ctor_get(x_1, 2); +lean_inc(x_13); lean_dec(x_1); -x_12 = lean_apply_6(x_11, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_12) == 0) +x_14 = lean_apply_6(x_13, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_14) == 0) { -uint8_t x_13; -x_13 = !lean_is_exclusive(x_12); -if (x_13 == 0) +uint8_t x_15; +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 0) { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_14 = lean_ctor_get(x_12, 0); -x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__7___closed__2; -x_16 = l_Lean_Expr_const___override(x_15, x_2); -x_17 = l_Lean_mkApp3(x_16, x_3, x_4, x_14); -lean_ctor_set(x_12, 0, x_17); -return x_12; +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_16 = lean_ctor_get(x_14, 0); +x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__1___closed__2; +x_18 = l_Lean_Expr_const___override(x_17, x_2); +x_19 = l_Lean_mkApp5(x_18, x_3, x_4, x_5, x_6, x_16); +lean_ctor_set(x_14, 0, x_19); +return x_14; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_18 = lean_ctor_get(x_12, 0); -x_19 = lean_ctor_get(x_12, 1); -lean_inc(x_19); -lean_inc(x_18); -lean_dec(x_12); -x_20 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__7___closed__2; -x_21 = l_Lean_Expr_const___override(x_20, x_2); -x_22 = l_Lean_mkApp3(x_21, x_3, x_4, x_18); -x_23 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_23, 0, x_22); -lean_ctor_set(x_23, 1, x_19); -return x_23; +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_20 = lean_ctor_get(x_14, 0); +x_21 = lean_ctor_get(x_14, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_14); +x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__1___closed__2; +x_23 = l_Lean_Expr_const___override(x_22, x_2); +x_24 = l_Lean_mkApp5(x_23, x_3, x_4, x_5, x_6, x_20); +x_25 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_25, 0, x_24); +lean_ctor_set(x_25, 1, x_21); +return x_25; } } else { -uint8_t x_24; +uint8_t x_26; +lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_24 = !lean_is_exclusive(x_12); -if (x_24 == 0) +x_26 = !lean_is_exclusive(x_14); +if (x_26 == 0) { -return x_12; +return x_14; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_12, 0); -x_26 = lean_ctor_get(x_12, 1); -lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_12); -x_27 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_26); -return x_27; -} -} -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("ofBool", 6, 6); -return x_1; +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_14, 0); +x_28 = lean_ctor_get(x_14, 1); +lean_inc(x_28); +lean_inc(x_27); +lean_dec(x_14); +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_27); +lean_ctor_set(x_29, 1, x_28); +return x_29; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__2; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__1; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__2___closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__2; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__6; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__4() { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__2; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__5() { -_start: +lean_object* x_9; +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_1); +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(x_1, x_3, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_9) == 0) { -lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(1u); -x_2 = l_Lean_mkNatLit(x_1); -return x_2; -} +lean_object* x_10; +x_10 = lean_ctor_get(x_9, 0); +lean_inc(x_10); +if (lean_obj_tag(x_10) == 0) +{ +uint8_t x_11; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_11 = !lean_is_exclusive(x_9); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; +x_12 = lean_ctor_get(x_9, 0); +lean_dec(x_12); +x_13 = lean_box(0); +lean_ctor_set(x_9, 0, x_13); +return x_9; } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__6() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(0u); -x_2 = l_Lean_mkNatLit(x_1); -return x_2; +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_9, 1); +lean_inc(x_14); +lean_dec(x_9); +x_15 = lean_box(0); +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_16, 1, x_14); +return x_16; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_9 = lean_box(0); -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__3; -lean_inc(x_1); -x_11 = l_Lean_Expr_app___override(x_10, x_1); -x_12 = lean_unsigned_to_nat(1u); -x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom(x_11, x_12, x_3, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_13) == 0) -{ -uint8_t x_14; -x_14 = !lean_is_exclusive(x_13); -if (x_14 == 0) +else { -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_15 = lean_ctor_get(x_13, 0); -x_16 = lean_ctor_get(x_15, 0); -lean_inc(x_16); -x_17 = lean_ctor_get(x_15, 1); +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_9, 1); lean_inc(x_17); -x_18 = lean_ctor_get(x_15, 3); -lean_inc(x_18); -x_19 = lean_unsigned_to_nat(0u); -lean_inc(x_16); -x_20 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_20, 0, x_16); -lean_ctor_set(x_20, 1, x_17); -lean_ctor_set(x_20, 2, x_19); -x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__4; -x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__5; -x_23 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__6; +lean_dec(x_9); +x_18 = lean_ctor_get(x_10, 0); lean_inc(x_18); -x_24 = l_Lean_mkApp3(x_21, x_22, x_18, x_23); -x_25 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_25, 0, x_16); -lean_closure_set(x_25, 1, x_18); -x_26 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__7), 10, 3); -lean_closure_set(x_26, 0, x_15); -lean_closure_set(x_26, 1, x_9); -lean_closure_set(x_26, 2, x_1); -x_27 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_27, 0, x_25); -lean_closure_set(x_27, 1, x_26); -x_28 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_28, 0, x_20); -lean_ctor_set(x_28, 1, x_27); -lean_ctor_set(x_28, 2, x_24); -x_29 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_29, 0, x_28); -lean_ctor_set(x_13, 0, x_29); -return x_13; +lean_dec(x_10); +x_19 = l_Lean_Meta_getNatValue_x3f(x_2, x_4, x_5, x_6, x_7, x_17); +if (lean_obj_tag(x_19) == 0) +{ +lean_object* x_20; +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +if (lean_obj_tag(x_20) == 0) +{ +uint8_t x_21; +lean_dec(x_18); +lean_dec(x_2); +lean_dec(x_1); +x_21 = !lean_is_exclusive(x_19); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; +x_22 = lean_ctor_get(x_19, 0); +lean_dec(x_22); +x_23 = lean_box(0); +lean_ctor_set(x_19, 0, x_23); +return x_19; } else { -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_30 = lean_ctor_get(x_13, 0); -x_31 = lean_ctor_get(x_13, 1); +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_19, 1); +lean_inc(x_24); +lean_dec(x_19); +x_25 = lean_box(0); +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_24); +return x_26; +} +} +else +{ +uint8_t x_27; +x_27 = !lean_is_exclusive(x_19); +if (x_27 == 0) +{ +lean_object* x_28; uint8_t x_29; +x_28 = lean_ctor_get(x_19, 0); +lean_dec(x_28); +x_29 = !lean_is_exclusive(x_20); +if (x_29 == 0) +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_30 = lean_ctor_get(x_20, 0); +x_31 = lean_ctor_get(x_18, 0); lean_inc(x_31); -lean_inc(x_30); -lean_dec(x_13); -x_32 = lean_ctor_get(x_30, 0); +x_32 = lean_ctor_get(x_18, 1); lean_inc(x_32); -x_33 = lean_ctor_get(x_30, 1); +x_33 = lean_ctor_get(x_18, 3); lean_inc(x_33); -x_34 = lean_ctor_get(x_30, 3); -lean_inc(x_34); -x_35 = lean_unsigned_to_nat(0u); -lean_inc(x_32); -x_36 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_36, 0, x_32); -lean_ctor_set(x_36, 1, x_33); -lean_ctor_set(x_36, 2, x_35); -x_37 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__4; -x_38 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__5; -x_39 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__6; -lean_inc(x_34); -x_40 = l_Lean_mkApp3(x_37, x_38, x_34, x_39); -x_41 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_41, 0, x_32); -lean_closure_set(x_41, 1, x_34); -x_42 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__7), 10, 3); -lean_closure_set(x_42, 0, x_30); -lean_closure_set(x_42, 1, x_9); -lean_closure_set(x_42, 2, x_1); -x_43 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_43, 0, x_41); -lean_closure_set(x_43, 1, x_42); -x_44 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_44, 0, x_36); -lean_ctor_set(x_44, 1, x_43); -lean_ctor_set(x_44, 2, x_40); -x_45 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_45, 0, x_44); -x_46 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_46, 0, x_45); -lean_ctor_set(x_46, 1, x_31); -return x_46; +lean_inc(x_31); +x_34 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_34, 0, x_31); +lean_ctor_set(x_34, 1, x_32); +lean_ctor_set(x_34, 2, x_30); +x_35 = lean_box(0); +lean_inc(x_31); +x_36 = l_Lean_mkNatLit(x_31); +x_37 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__2___closed__1; +lean_inc(x_2); +lean_inc(x_33); +lean_inc(x_36); +x_38 = l_Lean_mkApp3(x_37, x_36, x_33, x_2); +x_39 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_39, 0, x_31); +lean_closure_set(x_39, 1, x_33); +x_40 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__1), 12, 5); +lean_closure_set(x_40, 0, x_18); +lean_closure_set(x_40, 1, x_35); +lean_closure_set(x_40, 2, x_2); +lean_closure_set(x_40, 3, x_36); +lean_closure_set(x_40, 4, x_1); +x_41 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_41, 0, x_39); +lean_closure_set(x_41, 1, x_40); +x_42 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_42, 0, x_34); +lean_ctor_set(x_42, 1, x_41); +lean_ctor_set(x_42, 2, x_38); +lean_ctor_set(x_20, 0, x_42); +return x_19; +} +else +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; +x_43 = lean_ctor_get(x_20, 0); +lean_inc(x_43); +lean_dec(x_20); +x_44 = lean_ctor_get(x_18, 0); +lean_inc(x_44); +x_45 = lean_ctor_get(x_18, 1); +lean_inc(x_45); +x_46 = lean_ctor_get(x_18, 3); +lean_inc(x_46); +lean_inc(x_44); +x_47 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_47, 0, x_44); +lean_ctor_set(x_47, 1, x_45); +lean_ctor_set(x_47, 2, x_43); +x_48 = lean_box(0); +lean_inc(x_44); +x_49 = l_Lean_mkNatLit(x_44); +x_50 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__2___closed__1; +lean_inc(x_2); +lean_inc(x_46); +lean_inc(x_49); +x_51 = l_Lean_mkApp3(x_50, x_49, x_46, x_2); +x_52 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_52, 0, x_44); +lean_closure_set(x_52, 1, x_46); +x_53 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__1), 12, 5); +lean_closure_set(x_53, 0, x_18); +lean_closure_set(x_53, 1, x_48); +lean_closure_set(x_53, 2, x_2); +lean_closure_set(x_53, 3, x_49); +lean_closure_set(x_53, 4, x_1); +x_54 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_54, 0, x_52); +lean_closure_set(x_54, 1, x_53); +x_55 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_55, 0, x_47); +lean_ctor_set(x_55, 1, x_54); +lean_ctor_set(x_55, 2, x_51); +x_56 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_56, 0, x_55); +lean_ctor_set(x_19, 0, x_56); +return x_19; +} +} +else +{ +lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; +x_57 = lean_ctor_get(x_19, 1); +lean_inc(x_57); +lean_dec(x_19); +x_58 = lean_ctor_get(x_20, 0); +lean_inc(x_58); +if (lean_is_exclusive(x_20)) { + lean_ctor_release(x_20, 0); + x_59 = x_20; +} else { + lean_dec_ref(x_20); + x_59 = lean_box(0); +} +x_60 = lean_ctor_get(x_18, 0); +lean_inc(x_60); +x_61 = lean_ctor_get(x_18, 1); +lean_inc(x_61); +x_62 = lean_ctor_get(x_18, 3); +lean_inc(x_62); +lean_inc(x_60); +x_63 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_63, 0, x_60); +lean_ctor_set(x_63, 1, x_61); +lean_ctor_set(x_63, 2, x_58); +x_64 = lean_box(0); +lean_inc(x_60); +x_65 = l_Lean_mkNatLit(x_60); +x_66 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__2___closed__1; +lean_inc(x_2); +lean_inc(x_62); +lean_inc(x_65); +x_67 = l_Lean_mkApp3(x_66, x_65, x_62, x_2); +x_68 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_68, 0, x_60); +lean_closure_set(x_68, 1, x_62); +x_69 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__1), 12, 5); +lean_closure_set(x_69, 0, x_18); +lean_closure_set(x_69, 1, x_64); +lean_closure_set(x_69, 2, x_2); +lean_closure_set(x_69, 3, x_65); +lean_closure_set(x_69, 4, x_1); +x_70 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_70, 0, x_68); +lean_closure_set(x_70, 1, x_69); +x_71 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_71, 0, x_63); +lean_ctor_set(x_71, 1, x_70); +lean_ctor_set(x_71, 2, x_67); +if (lean_is_scalar(x_59)) { + x_72 = lean_alloc_ctor(1, 1, 0); +} else { + x_72 = x_59; +} +lean_ctor_set(x_72, 0, x_71); +x_73 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_73, 0, x_72); +lean_ctor_set(x_73, 1, x_57); +return x_73; +} +} +} +else +{ +uint8_t x_74; +lean_dec(x_18); +lean_dec(x_2); +lean_dec(x_1); +x_74 = !lean_is_exclusive(x_19); +if (x_74 == 0) +{ +return x_19; +} +else +{ +lean_object* x_75; lean_object* x_76; lean_object* x_77; +x_75 = lean_ctor_get(x_19, 0); +x_76 = lean_ctor_get(x_19, 1); +lean_inc(x_76); +lean_inc(x_75); +lean_dec(x_19); +x_77 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_77, 0, x_75); +lean_ctor_set(x_77, 1, x_76); +return x_77; +} +} } } else { -uint8_t x_47; +uint8_t x_78; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); lean_dec(x_1); -x_47 = !lean_is_exclusive(x_13); -if (x_47 == 0) +x_78 = !lean_is_exclusive(x_9); +if (x_78 == 0) { -return x_13; +return x_9; } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_ctor_get(x_13, 0); -x_49 = lean_ctor_get(x_13, 1); -lean_inc(x_49); -lean_inc(x_48); -lean_dec(x_13); -x_50 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_50, 0, x_48); -lean_ctor_set(x_50, 1, x_49); -return x_50; +lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_79 = lean_ctor_get(x_9, 0); +x_80 = lean_ctor_get(x_9, 1); +lean_inc(x_80); +lean_inc(x_79); +lean_dec(x_9); +x_81 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_81, 0, x_79); +lean_ctor_set(x_81, 1, x_80); +return x_81; } } } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__3___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("Bool", 4, 4); +x_1 = lean_mk_string_unchecked("ult_congr", 9, 9); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__3___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__3; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__4; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__5; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__3___closed__1; +x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +uint8_t x_9; lean_object* x_10; lean_object* x_11; +x_9 = 1; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__3___closed__2; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection(x_1, x_2, x_9, x_10, x_3, x_4, x_5, x_6, x_7, x_8); +return x_11; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__4___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("beq_congr", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__4___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__3; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__4; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__5; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__4___closed__1; +x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +uint8_t x_10; lean_object* x_11; lean_object* x_12; +x_10 = 0; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__4___closed__2; +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection(x_1, x_2, x_10, x_11, x_4, x_5, x_6, x_7, x_8, x_9); +return x_12; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__5___closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__5; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_9; -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_1); -x_9 = lean_infer_type(x_1, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_9) == 0) -{ -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; -x_10 = lean_ctor_get(x_9, 0); -lean_inc(x_10); -x_11 = lean_ctor_get(x_9, 1); -lean_inc(x_11); -lean_dec(x_9); -x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__6___closed__1; -x_13 = l_Lean_Expr_cleanupAnnotations(x_10); -x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9___closed__2; -x_15 = l_Lean_Expr_isConstOf(x_13, x_14); -lean_dec(x_13); -if (x_15 == 0) +lean_object* x_10; lean_object* x_11; uint8_t x_12; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__1; +x_11 = l_Lean_Expr_cleanupAnnotations(x_1); +x_12 = l_Lean_Expr_isApp(x_11); +if (x_12 == 0) { -lean_object* x_16; lean_object* x_17; -lean_dec(x_1); -x_16 = lean_box(0); -x_17 = lean_apply_7(x_12, x_16, x_3, x_4, x_5, x_6, x_7, x_11); -return x_17; +lean_object* x_13; lean_object* x_14; +lean_dec(x_11); +lean_dec(x_3); +lean_dec(x_2); +x_13 = lean_box(0); +x_14 = lean_apply_7(x_10, x_13, x_4, x_5, x_6, x_7, x_8, x_9); +return x_14; } else { +lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_15 = l_Lean_Expr_appFnCleanup(x_11, lean_box(0)); +x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__5___closed__1; +x_17 = l_Lean_Expr_isConstOf(x_15, x_16); +lean_dec(x_15); +if (x_17 == 0) +{ lean_object* x_18; lean_object* x_19; +lean_dec(x_3); +lean_dec(x_2); x_18 = lean_box(0); -x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8(x_1, x_18, x_3, x_4, x_5, x_6, x_7, x_11); +x_19 = lean_apply_7(x_10, x_18, x_4, x_5, x_6, x_7, x_8, x_9); return x_19; } -} -else -{ -uint8_t x_20; -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_20 = !lean_is_exclusive(x_9); -if (x_20 == 0) -{ -return x_9; -} else { -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_9, 0); -x_22 = lean_ctor_get(x_9, 1); -lean_inc(x_22); -lean_inc(x_21); -lean_dec(x_9); -x_23 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_23, 0, x_21); -lean_ctor_set(x_23, 1, x_22); -return x_23; +lean_object* x_20; lean_object* x_21; +x_20 = lean_box(0); +x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__4(x_2, x_3, x_20, x_4, x_5, x_6, x_7, x_8, x_9); +return x_21; } } } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2), 8, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__2), 8, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__2() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__3), 8, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__3), 8, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__3() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__6), 9, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__5), 9, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__2; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__1; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__5; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__5; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__2; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__12; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__5; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__8; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__6() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__6() { _start: { lean_object* x_1; @@ -1852,7 +1875,7 @@ x_1 = lean_mk_string_unchecked("BEq", 3, 3); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__7() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__7() { _start: { lean_object* x_1; @@ -1860,184 +1883,264 @@ x_1 = lean_mk_string_unchecked("beq", 3, 3); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__8() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__6; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__7; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__6; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__7; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; -lean_inc(x_1); +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; x_8 = l_Lean_Meta_instantiateMVarsIfMVarApp(x_1, x_3, x_4, x_5, x_6, x_7); x_9 = lean_ctor_get(x_8, 0); lean_inc(x_9); x_10 = lean_ctor_get(x_8, 1); lean_inc(x_10); lean_dec(x_8); -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__1; -x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__2; -x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__3; -x_14 = l_Lean_Expr_cleanupAnnotations(x_9); -x_15 = l_Lean_Expr_isApp(x_14); -if (x_15 == 0) -{ -lean_object* x_16; lean_object* x_17; -lean_dec(x_14); -x_16 = lean_box(0); -x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9(x_1, x_16, x_2, x_3, x_4, x_5, x_6, x_10); -return x_17; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__1; +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__2; +x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__3; +x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__1; +x_15 = l_Lean_Expr_cleanupAnnotations(x_9); +x_16 = l_Lean_Expr_isApp(x_15); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; +lean_dec(x_15); +x_17 = lean_box(0); +x_18 = lean_apply_7(x_14, x_17, x_2, x_3, x_4, x_5, x_6, x_10); +return x_18; } else { -lean_object* x_18; lean_object* x_19; uint8_t x_20; -x_18 = l_Lean_Expr_appArg(x_14, lean_box(0)); -x_19 = l_Lean_Expr_appFnCleanup(x_14, lean_box(0)); -x_20 = l_Lean_Expr_isApp(x_19); -if (x_20 == 0) +lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_19 = l_Lean_Expr_appArg(x_15, lean_box(0)); +x_20 = l_Lean_Expr_appFnCleanup(x_15, lean_box(0)); +x_21 = l_Lean_Expr_isApp(x_20); +if (x_21 == 0) { -lean_object* x_21; lean_object* x_22; +lean_object* x_22; lean_object* x_23; +lean_dec(x_20); lean_dec(x_19); -lean_dec(x_18); -x_21 = lean_box(0); -x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9(x_1, x_21, x_2, x_3, x_4, x_5, x_6, x_10); -return x_22; +x_22 = lean_box(0); +x_23 = lean_apply_7(x_14, x_22, x_2, x_3, x_4, x_5, x_6, x_10); +return x_23; } else { -lean_object* x_23; lean_object* x_24; uint8_t x_25; -x_23 = l_Lean_Expr_appArg(x_19, lean_box(0)); -x_24 = l_Lean_Expr_appFnCleanup(x_19, lean_box(0)); -x_25 = l_Lean_Expr_isApp(x_24); -if (x_25 == 0) +lean_object* x_24; lean_object* x_25; uint8_t x_26; +x_24 = l_Lean_Expr_appArg(x_20, lean_box(0)); +x_25 = l_Lean_Expr_appFnCleanup(x_20, lean_box(0)); +x_26 = l_Lean_Expr_isApp(x_25); +if (x_26 == 0) { -lean_object* x_26; lean_object* x_27; +lean_object* x_27; lean_object* x_28; +lean_dec(x_25); lean_dec(x_24); -lean_dec(x_23); -lean_dec(x_18); -x_26 = lean_box(0); -x_27 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9(x_1, x_26, x_2, x_3, x_4, x_5, x_6, x_10); -return x_27; +lean_dec(x_19); +x_27 = lean_box(0); +x_28 = lean_apply_7(x_14, x_27, x_2, x_3, x_4, x_5, x_6, x_10); +return x_28; } else { -lean_object* x_28; lean_object* x_29; uint8_t x_30; -x_28 = l_Lean_Expr_appFnCleanup(x_24, lean_box(0)); -x_29 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__4; -x_30 = l_Lean_Expr_isConstOf(x_28, x_29); -if (x_30 == 0) -{ -lean_object* x_31; uint8_t x_32; -x_31 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__5; -x_32 = l_Lean_Expr_isConstOf(x_28, x_31); -if (x_32 == 0) +lean_object* x_29; lean_object* x_30; uint8_t x_31; +x_29 = l_Lean_Expr_appFnCleanup(x_25, lean_box(0)); +x_30 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__4; +x_31 = l_Lean_Expr_isConstOf(x_29, x_30); +if (x_31 == 0) { -uint8_t x_33; -x_33 = l_Lean_Expr_isApp(x_28); +lean_object* x_32; uint8_t x_33; +x_32 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__5; +x_33 = l_Lean_Expr_isConstOf(x_29, x_32); if (x_33 == 0) { -lean_object* x_34; lean_object* x_35; -lean_dec(x_28); -lean_dec(x_23); -lean_dec(x_18); -x_34 = lean_box(0); -x_35 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9(x_1, x_34, x_2, x_3, x_4, x_5, x_6, x_10); -return x_35; -} -else -{ -lean_object* x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; -x_36 = l_Lean_Expr_appArg(x_28, lean_box(0)); -x_37 = l_Lean_Expr_appFnCleanup(x_28, lean_box(0)); -x_38 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__8; -x_39 = l_Lean_Expr_isConstOf(x_37, x_38); -lean_dec(x_37); -if (x_39 == 0) +uint8_t x_34; +x_34 = l_Lean_Expr_isApp(x_29); +if (x_34 == 0) { -lean_object* x_40; lean_object* x_41; -lean_dec(x_36); -lean_dec(x_23); -lean_dec(x_18); -x_40 = lean_box(0); -x_41 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9(x_1, x_40, x_2, x_3, x_4, x_5, x_6, x_10); -return x_41; +lean_object* x_35; lean_object* x_36; +lean_dec(x_29); +lean_dec(x_24); +lean_dec(x_19); +x_35 = lean_box(0); +x_36 = lean_apply_7(x_14, x_35, x_2, x_3, x_4, x_5, x_6, x_10); +return x_36; } else { -lean_object* x_42; -lean_dec(x_1); -x_42 = lean_apply_9(x_13, x_36, x_23, x_18, x_2, x_3, x_4, x_5, x_6, x_10); +lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; +x_37 = l_Lean_Expr_appArg(x_29, lean_box(0)); +x_38 = l_Lean_Expr_appFnCleanup(x_29, lean_box(0)); +x_39 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__8; +x_40 = l_Lean_Expr_isConstOf(x_38, x_39); +lean_dec(x_38); +if (x_40 == 0) +{ +lean_object* x_41; lean_object* x_42; +lean_dec(x_37); +lean_dec(x_24); +lean_dec(x_19); +x_41 = lean_box(0); +x_42 = lean_apply_7(x_14, x_41, x_2, x_3, x_4, x_5, x_6, x_10); return x_42; } -} -} else { lean_object* x_43; -lean_dec(x_28); -lean_dec(x_1); -x_43 = lean_apply_8(x_12, x_23, x_18, x_2, x_3, x_4, x_5, x_6, x_10); +x_43 = lean_apply_9(x_13, x_37, x_24, x_19, x_2, x_3, x_4, x_5, x_6, x_10); return x_43; } } +} else { lean_object* x_44; -lean_dec(x_28); -lean_dec(x_1); -x_44 = lean_apply_8(x_11, x_23, x_18, x_2, x_3, x_4, x_5, x_6, x_10); +lean_dec(x_29); +x_44 = lean_apply_8(x_12, x_24, x_19, x_2, x_3, x_4, x_5, x_6, x_10); return x_44; } } +else +{ +lean_object* x_45; +lean_dec(x_29); +x_45 = lean_apply_8(x_11, x_24, x_19, x_2, x_3, x_4, x_5, x_6, x_10); +return x_45; +} } } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { lean_object* x_10; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_3); return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; -x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +if (lean_obj_tag(x_8) == 0) +{ +lean_object* x_9; +x_9 = lean_ctor_get(x_8, 0); +lean_inc(x_9); +if (lean_obj_tag(x_9) == 0) +{ +lean_object* x_10; lean_object* x_11; +x_10 = lean_ctor_get(x_8, 1); +lean_inc(x_10); +lean_dec(x_8); +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom(x_1, x_2, x_3, x_4, x_5, x_6, x_10); +return x_11; +} +else +{ +uint8_t x_12; lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); +x_12 = !lean_is_exclusive(x_8); +if (x_12 == 0) +{ +lean_object* x_13; uint8_t x_14; +x_13 = lean_ctor_get(x_8, 0); +lean_dec(x_13); +x_14 = !lean_is_exclusive(x_9); +if (x_14 == 0) +{ +return x_8; +} +else +{ +lean_object* x_15; lean_object* x_16; +x_15 = lean_ctor_get(x_9, 0); +lean_inc(x_15); +lean_dec(x_9); +x_16 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_8, 0, x_16); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: +else { -lean_object* x_9; -x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_2); -return x_9; +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_17 = lean_ctor_get(x_8, 1); +lean_inc(x_17); +lean_dec(x_8); +x_18 = lean_ctor_get(x_9, 0); +lean_inc(x_18); +if (lean_is_exclusive(x_9)) { + lean_ctor_release(x_9, 0); + x_19 = x_9; +} else { + lean_dec_ref(x_9); + x_19 = lean_box(0); +} +if (lean_is_scalar(x_19)) { + x_20 = lean_alloc_ctor(1, 1, 0); +} else { + x_20 = x_19; +} +lean_ctor_set(x_20, 0, x_18); +x_21 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_21, 0, x_20); +lean_ctor_set(x_21, 1, x_17); +return x_21; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: +} +else { -lean_object* x_9; -x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +uint8_t x_22; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); -return x_9; +lean_dec(x_1); +x_22 = !lean_is_exclusive(x_8); +if (x_22 == 0) +{ +return x_8; +} +else +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_8, 0); +x_24 = lean_ctor_get(x_8, 1); +lean_inc(x_24); +lean_inc(x_23); +lean_dec(x_8); +x_25 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +return x_25; +} +} } } lean_object* initialize_Lean_Elab_Tactic_BVDecide_Frontend_BVDecide_ReifiedBVExpr(uint8_t builtin, lean_object*); @@ -2049,6 +2152,44 @@ _G_initialized = true; res = initialize_Lean_Elab_Tactic_BVDecide_Frontend_BVDecide_ReifiedBVExpr(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__7); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__7); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__8(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__8); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__9 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__9(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__9); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__3); l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__1(); lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__1); l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__2(); @@ -2069,76 +2210,38 @@ l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed_ lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__9); l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__10 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__10(); lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__10); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__11 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__11(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__11); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__12 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__12(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__12); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__13 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__13(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__13); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__14 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__14(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__14); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__3___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__3___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__3___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__3___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__3___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__3___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__4___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__4___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__4___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__4___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__4___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__4___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__6___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__6___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__6___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__6___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__6___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__6___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__7___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__7___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__7___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__7___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__7___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__7___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__6); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__6); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__7); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__8(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__8); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__1___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__1___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__2___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__2___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__3___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__3___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__3___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__3___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__3___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__4___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__4___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__4___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__4___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__4___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__4___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__5___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__5___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__5___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__7); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__8(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__8); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/SatAtBVLogical.c b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/SatAtBVLogical.c index 1c8757fb750f..387d7ba4acfe 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/SatAtBVLogical.c +++ b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/SatAtBVLogical.c @@ -16,6 +16,7 @@ extern "C" { lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_of___lambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_of___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goOrAtom(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_of___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_of___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkTrans(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -50,7 +51,6 @@ static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_and___la lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_and___lambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_and(lean_object*, lean_object*); -lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_and___closed__7; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_and___lambda__1___closed__3; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_proveFalse___closed__2; @@ -73,10 +73,10 @@ lean_object* l_Lean_Meta_instantiateMVarsIfMVarApp(lean_object*, lean_object*, l static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_and___closed__5; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_and___closed__9; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_of___lambda__4___closed__1; +lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_of(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_proveFalse(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_of___lambda__1___closed__2; lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_of___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -189,7 +189,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_of_ { lean_object* x_10; lean_inc(x_1); -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of(x_1, x_4, x_5, x_6, x_7, x_8, x_9); +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goOrAtom(x_1, x_4, x_5, x_6, x_7, x_8, x_9); if (lean_obj_tag(x_10) == 0) { lean_object* x_11; @@ -546,7 +546,7 @@ lean_inc(x_12); x_13 = lean_ctor_get(x_11, 1); lean_inc(x_13); lean_dec(x_11); -x_14 = l_Lean_instantiateMVars___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom___spec__1(x_12, x_2, x_3, x_4, x_5, x_6, x_13); +x_14 = l_Lean_instantiateMVars___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom___spec__1(x_12, x_2, x_3, x_4, x_5, x_6, x_13); x_15 = lean_ctor_get(x_14, 0); lean_inc(x_15); x_16 = lean_ctor_get(x_14, 1); diff --git a/stage0/stdlib/Lean/Elab/Tactic/BuiltinTactic.c b/stage0/stdlib/Lean/Elab/Tactic/BuiltinTactic.c index cabd58b36fb0..6a7e3ea33346 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/BuiltinTactic.c +++ b/stage0/stdlib/Lean/Elab/Tactic/BuiltinTactic.c @@ -95,7 +95,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_withRestoreOrSaveFull___at_Lean_Elab_Tactic LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at_Lean_Elab_Tactic_evalSepTactics_goEven___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalIntroMatch__1___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalTraceState_declRange__1___closed__4; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___boxed(lean_object**); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalClear_declRange__1___closed__6; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_evalOpen___spec__35___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalAnyGoals_declRange__1___closed__5; @@ -929,10 +929,10 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSleep_declRange__1( static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalFail_declRange__1___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalRunTac_declRange__1___closed__7; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalIntroMatch_declRange__1(lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalSepTactics(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_withAlwaysResolvedPromise___at_Lean_Elab_Tactic_evalSepTactics_goEven___spec__18(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalCase___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalCase___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalWithAnnotateState__1___closed__9; LEAN_EXPORT lean_object* l_Lean_getRefPos___at_Lean_Elab_Tactic_evalOpen___spec__38___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalLeft_declRange__1___closed__1; @@ -1189,7 +1189,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalAllGoals___boxed(lean_object*, l LEAN_EXPORT lean_object* l_Lean_Elab_Term_withRestoreOrSaveFull___at_Lean_Elab_Tactic_evalSepTactics_goEven___spec__10___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Tactic_evalOpen___spec__3___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalRotateLeft__1___closed__4; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalCase___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalCase___lambda__2___boxed(lean_object**); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalCase(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_renameInaccessibles___spec__14(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalRefl_declRange__1(lean_object*); @@ -1352,7 +1352,7 @@ static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalOpen__1___closed__2; LEAN_EXPORT lean_object* l_Lean_resolveNamespace___at_Lean_Elab_Tactic_evalOpen___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_evalSubstVars___rarg___closed__1; lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_local_ctx_num_indices(lean_object*); static lean_object* l_Lean_Elab_Tactic_evalRunTac___closed__10; LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at_Lean_Elab_Tactic_evalSepTactics_goEven___spec__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1413,7 +1413,7 @@ lean_object* l_Lean_MVarId_replaceLocalDeclDefEq(lean_object*, lean_object*, lea static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalClear_declRange__1___closed__4; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_renameInaccessibles___spec__16(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Tactic_evalOpen___spec__28___closed__2; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase___spec__6___boxed(lean_object**); lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalTacticSeqBracketed__1___closed__4; uint8_t lean_nat_dec_le(lean_object*, lean_object*); @@ -40600,14 +40600,15 @@ return x_40; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, size_t x_6, size_t x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { _start: { -uint8_t x_17; -x_17 = lean_usize_dec_lt(x_6, x_5); -if (x_17 == 0) +uint8_t x_18; +x_18 = lean_usize_dec_lt(x_7, x_6); +if (x_18 == 0) { -lean_object* x_18; +lean_object* x_19; +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -40615,72 +40616,73 @@ lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_7); -lean_ctor_set(x_18, 1, x_16); -return x_18; +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_8); +lean_ctor_set(x_19, 1, x_17); +return x_19; } else { -lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; -x_19 = lean_array_uget(x_4, x_6); -x_29 = lean_ctor_get(x_7, 0); -lean_inc(x_29); -x_30 = lean_ctor_get(x_7, 1); +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; +x_20 = lean_array_uget(x_5, x_7); +x_30 = lean_ctor_get(x_8, 0); lean_inc(x_30); -x_31 = lean_ctor_get(x_7, 2); +x_31 = lean_ctor_get(x_8, 1); lean_inc(x_31); -x_32 = lean_nat_dec_lt(x_30, x_31); -if (x_32 == 0) +x_32 = lean_ctor_get(x_8, 2); +lean_inc(x_32); +x_33 = lean_nat_dec_lt(x_31, x_32); +if (x_33 == 0) { -lean_object* x_33; +lean_object* x_34; +lean_dec(x_32); lean_dec(x_31); lean_dec(x_30); -lean_dec(x_29); -lean_dec(x_19); -x_33 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_33, 0, x_7); -x_20 = x_33; -x_21 = x_16; -goto block_28; +lean_dec(x_20); +x_34 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_34, 0, x_8); +x_21 = x_34; +x_22 = x_17; +goto block_29; } else { -uint8_t x_34; -x_34 = !lean_is_exclusive(x_7); -if (x_34 == 0) +uint8_t x_35; +x_35 = !lean_is_exclusive(x_8); +if (x_35 == 0) { -lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_35 = lean_ctor_get(x_7, 2); -lean_dec(x_35); -x_36 = lean_ctor_get(x_7, 1); +lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_36 = lean_ctor_get(x_8, 2); lean_dec(x_36); -x_37 = lean_ctor_get(x_7, 0); +x_37 = lean_ctor_get(x_8, 1); lean_dec(x_37); -x_38 = lean_array_fget(x_29, x_30); -x_39 = lean_unsigned_to_nat(1u); -x_40 = lean_nat_add(x_30, x_39); -lean_dec(x_30); -lean_ctor_set(x_7, 1, x_40); -x_41 = l___private_Lean_Elab_Tactic_BuiltinTactic_0__Lean_Elab_Tactic_getCaseGoals(x_19, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_41) == 0) +x_38 = lean_ctor_get(x_8, 0); +lean_dec(x_38); +x_39 = lean_array_fget(x_30, x_31); +x_40 = lean_unsigned_to_nat(1u); +x_41 = lean_nat_add(x_31, x_40); +lean_dec(x_31); +lean_ctor_set(x_8, 1, x_41); +x_42 = l___private_Lean_Elab_Tactic_BuiltinTactic_0__Lean_Elab_Tactic_getCaseGoals(x_20, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +if (lean_obj_tag(x_42) == 0) { -lean_object* x_42; lean_object* x_43; uint8_t x_44; -x_42 = lean_ctor_get(x_41, 0); -lean_inc(x_42); -x_43 = lean_ctor_get(x_41, 1); +lean_object* x_43; lean_object* x_44; uint8_t x_45; +x_43 = lean_ctor_get(x_42, 0); lean_inc(x_43); -lean_dec(x_41); -x_44 = !lean_is_exclusive(x_42); -if (x_44 == 0) +x_44 = lean_ctor_get(x_42, 1); +lean_inc(x_44); +lean_dec(x_42); +x_45 = !lean_is_exclusive(x_43); +if (x_45 == 0) { -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_42, 0); -x_46 = lean_ctor_get(x_42, 1); +lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_46 = lean_ctor_get(x_43, 0); +x_47 = lean_ctor_get(x_43, 1); +lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); @@ -40688,43 +40690,65 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); -x_47 = l_Lean_Elab_Tactic_renameInaccessibles(x_45, x_38, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_43); -if (lean_obj_tag(x_47) == 0) +x_48 = l_Lean_Elab_Tactic_renameInaccessibles(x_46, x_39, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_44); +if (lean_obj_tag(x_48) == 0) { -lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; -x_48 = lean_ctor_get(x_47, 0); -lean_inc(x_48); -x_49 = lean_ctor_get(x_47, 1); +lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; uint8_t x_53; +x_49 = lean_ctor_get(x_48, 0); lean_inc(x_49); -lean_dec(x_47); -x_50 = lean_box(0); -lean_inc(x_48); -lean_ctor_set_tag(x_42, 1); -lean_ctor_set(x_42, 1, x_50); -lean_ctor_set(x_42, 0, x_48); -x_51 = l_Lean_Elab_Tactic_setGoals(x_42, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_49); -x_52 = lean_ctor_get(x_51, 1); -lean_inc(x_52); -lean_dec(x_51); -x_53 = lean_box(0); -x_54 = l_Lean_MVarId_setTag(x_48, x_53, x_12, x_13, x_14, x_15, x_52); -x_55 = lean_ctor_get(x_54, 1); -lean_inc(x_55); -lean_dec(x_54); -x_56 = lean_unsigned_to_nat(3u); -x_57 = l_Lean_Elab_Tactic_evalWithAnnotateState___closed__1; -lean_inc(x_1); -x_58 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1), 12, 3); -lean_closure_set(x_58, 0, x_56); -lean_closure_set(x_58, 1, x_57); -lean_closure_set(x_58, 2, x_1); +x_50 = lean_ctor_get(x_48, 1); +lean_inc(x_50); +lean_dec(x_48); +x_51 = lean_box(0); +lean_inc(x_49); +lean_ctor_set_tag(x_43, 1); +lean_ctor_set(x_43, 1, x_51); +lean_ctor_set(x_43, 0, x_49); +x_52 = l_Lean_Elab_Tactic_setGoals(x_43, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_50); +x_53 = !lean_is_exclusive(x_52); +if (x_53 == 0) +{ +lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; uint8_t x_58; +x_54 = lean_ctor_get(x_52, 1); +x_55 = lean_ctor_get(x_52, 0); +lean_dec(x_55); +x_56 = lean_box(0); +x_57 = l_Lean_MVarId_setTag(x_49, x_56, x_13, x_14, x_15, x_16, x_54); +x_58 = !lean_is_exclusive(x_57); +if (x_58 == 0) +{ +lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; +x_59 = lean_ctor_get(x_57, 1); +x_60 = lean_ctor_get(x_57, 0); +lean_dec(x_60); +lean_inc(x_3); +lean_ctor_set_tag(x_57, 1); +lean_ctor_set(x_57, 1, x_51); +lean_ctor_set(x_57, 0, x_3); +lean_inc(x_2); +lean_ctor_set_tag(x_52, 1); +lean_ctor_set(x_52, 1, x_57); +lean_ctor_set(x_52, 0, x_2); +x_61 = lean_array_mk(x_52); +x_62 = lean_box(2); +x_63 = l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1___lambda__1___closed__2; +x_64 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_64, 0, x_62); +lean_ctor_set(x_64, 1, x_63); +lean_ctor_set(x_64, 2, x_61); +x_65 = lean_unsigned_to_nat(3u); +x_66 = l_Lean_Elab_Tactic_evalWithAnnotateState___closed__1; lean_inc(x_1); -x_59 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); -lean_closure_set(x_59, 0, x_1); -lean_closure_set(x_59, 1, x_58); -x_60 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_closeUsingOrAdmit), 10, 1); -lean_closure_set(x_60, 0, x_59); +x_67 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1), 12, 3); +lean_closure_set(x_67, 0, x_65); +lean_closure_set(x_67, 1, x_66); +lean_closure_set(x_67, 2, x_1); +x_68 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); +lean_closure_set(x_68, 0, x_64); +lean_closure_set(x_68, 1, x_67); +x_69 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_closeUsingOrAdmit), 10, 1); +lean_closure_set(x_69, 0, x_68); +lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); @@ -40732,31 +40756,31 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); +lean_inc(x_4); lean_inc(x_3); -lean_inc(x_2); -x_61 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalCase___spec__5(x_2, x_3, x_60, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_55); -if (lean_obj_tag(x_61) == 0) +x_70 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalCase___spec__5(x_3, x_4, x_69, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_59); +if (lean_obj_tag(x_70) == 0) { -lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; -x_62 = lean_ctor_get(x_61, 1); -lean_inc(x_62); -lean_dec(x_61); -x_63 = l_Lean_Elab_Tactic_setGoals(x_46, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_62); -x_64 = lean_ctor_get(x_63, 1); -lean_inc(x_64); -lean_dec(x_63); -x_65 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_65, 0, x_7); -x_20 = x_65; -x_21 = x_64; -goto block_28; +lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; +x_71 = lean_ctor_get(x_70, 1); +lean_inc(x_71); +lean_dec(x_70); +x_72 = l_Lean_Elab_Tactic_setGoals(x_47, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_71); +x_73 = lean_ctor_get(x_72, 1); +lean_inc(x_73); +lean_dec(x_72); +x_74 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_74, 0, x_8); +x_21 = x_74; +x_22 = x_73; +goto block_29; } else { -uint8_t x_66; -lean_dec(x_46); -lean_dec(x_7); +uint8_t x_75; +lean_dec(x_47); +lean_dec(x_8); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -40764,36 +40788,96 @@ lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_66 = !lean_is_exclusive(x_61); -if (x_66 == 0) +x_75 = !lean_is_exclusive(x_70); +if (x_75 == 0) { -return x_61; +return x_70; } else { -lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_67 = lean_ctor_get(x_61, 0); -x_68 = lean_ctor_get(x_61, 1); -lean_inc(x_68); -lean_inc(x_67); -lean_dec(x_61); -x_69 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_69, 0, x_67); -lean_ctor_set(x_69, 1, x_68); -return x_69; +lean_object* x_76; lean_object* x_77; lean_object* x_78; +x_76 = lean_ctor_get(x_70, 0); +x_77 = lean_ctor_get(x_70, 1); +lean_inc(x_77); +lean_inc(x_76); +lean_dec(x_70); +x_78 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_78, 0, x_76); +lean_ctor_set(x_78, 1, x_77); +return x_78; } } } else { -uint8_t x_70; -lean_free_object(x_42); -lean_dec(x_46); -lean_dec(x_7); +lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; +x_79 = lean_ctor_get(x_57, 1); +lean_inc(x_79); +lean_dec(x_57); +lean_inc(x_3); +x_80 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_80, 0, x_3); +lean_ctor_set(x_80, 1, x_51); +lean_inc(x_2); +lean_ctor_set_tag(x_52, 1); +lean_ctor_set(x_52, 1, x_80); +lean_ctor_set(x_52, 0, x_2); +x_81 = lean_array_mk(x_52); +x_82 = lean_box(2); +x_83 = l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1___lambda__1___closed__2; +x_84 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_84, 0, x_82); +lean_ctor_set(x_84, 1, x_83); +lean_ctor_set(x_84, 2, x_81); +x_85 = lean_unsigned_to_nat(3u); +x_86 = l_Lean_Elab_Tactic_evalWithAnnotateState___closed__1; +lean_inc(x_1); +x_87 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1), 12, 3); +lean_closure_set(x_87, 0, x_85); +lean_closure_set(x_87, 1, x_86); +lean_closure_set(x_87, 2, x_1); +x_88 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); +lean_closure_set(x_88, 0, x_84); +lean_closure_set(x_88, 1, x_87); +x_89 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_closeUsingOrAdmit), 10, 1); +lean_closure_set(x_89, 0, x_88); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_4); +lean_inc(x_3); +x_90 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalCase___spec__5(x_3, x_4, x_89, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_79); +if (lean_obj_tag(x_90) == 0) +{ +lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; +x_91 = lean_ctor_get(x_90, 1); +lean_inc(x_91); +lean_dec(x_90); +x_92 = l_Lean_Elab_Tactic_setGoals(x_47, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_91); +x_93 = lean_ctor_get(x_92, 1); +lean_inc(x_93); +lean_dec(x_92); +x_94 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_94, 0, x_8); +x_21 = x_94; +x_22 = x_93; +goto block_29; +} +else +{ +lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; +lean_dec(x_47); +lean_dec(x_8); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -40801,38 +40885,197 @@ lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_70 = !lean_is_exclusive(x_47); -if (x_70 == 0) +x_95 = lean_ctor_get(x_90, 0); +lean_inc(x_95); +x_96 = lean_ctor_get(x_90, 1); +lean_inc(x_96); +if (lean_is_exclusive(x_90)) { + lean_ctor_release(x_90, 0); + lean_ctor_release(x_90, 1); + x_97 = x_90; +} else { + lean_dec_ref(x_90); + x_97 = lean_box(0); +} +if (lean_is_scalar(x_97)) { + x_98 = lean_alloc_ctor(1, 2, 0); +} else { + x_98 = x_97; +} +lean_ctor_set(x_98, 0, x_95); +lean_ctor_set(x_98, 1, x_96); +return x_98; +} +} +} +else { -return x_47; +lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; +x_99 = lean_ctor_get(x_52, 1); +lean_inc(x_99); +lean_dec(x_52); +x_100 = lean_box(0); +x_101 = l_Lean_MVarId_setTag(x_49, x_100, x_13, x_14, x_15, x_16, x_99); +x_102 = lean_ctor_get(x_101, 1); +lean_inc(x_102); +if (lean_is_exclusive(x_101)) { + lean_ctor_release(x_101, 0); + lean_ctor_release(x_101, 1); + x_103 = x_101; +} else { + lean_dec_ref(x_101); + x_103 = lean_box(0); +} +lean_inc(x_3); +if (lean_is_scalar(x_103)) { + x_104 = lean_alloc_ctor(1, 2, 0); +} else { + x_104 = x_103; + lean_ctor_set_tag(x_104, 1); +} +lean_ctor_set(x_104, 0, x_3); +lean_ctor_set(x_104, 1, x_51); +lean_inc(x_2); +x_105 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_105, 0, x_2); +lean_ctor_set(x_105, 1, x_104); +x_106 = lean_array_mk(x_105); +x_107 = lean_box(2); +x_108 = l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1___lambda__1___closed__2; +x_109 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_109, 0, x_107); +lean_ctor_set(x_109, 1, x_108); +lean_ctor_set(x_109, 2, x_106); +x_110 = lean_unsigned_to_nat(3u); +x_111 = l_Lean_Elab_Tactic_evalWithAnnotateState___closed__1; +lean_inc(x_1); +x_112 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1), 12, 3); +lean_closure_set(x_112, 0, x_110); +lean_closure_set(x_112, 1, x_111); +lean_closure_set(x_112, 2, x_1); +x_113 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); +lean_closure_set(x_113, 0, x_109); +lean_closure_set(x_113, 1, x_112); +x_114 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_closeUsingOrAdmit), 10, 1); +lean_closure_set(x_114, 0, x_113); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_4); +lean_inc(x_3); +x_115 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalCase___spec__5(x_3, x_4, x_114, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_102); +if (lean_obj_tag(x_115) == 0) +{ +lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; +x_116 = lean_ctor_get(x_115, 1); +lean_inc(x_116); +lean_dec(x_115); +x_117 = l_Lean_Elab_Tactic_setGoals(x_47, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_116); +x_118 = lean_ctor_get(x_117, 1); +lean_inc(x_118); +lean_dec(x_117); +x_119 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_119, 0, x_8); +x_21 = x_119; +x_22 = x_118; +goto block_29; } else { -lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_71 = lean_ctor_get(x_47, 0); -x_72 = lean_ctor_get(x_47, 1); -lean_inc(x_72); -lean_inc(x_71); +lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_dec(x_47); -x_73 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_73, 0, x_71); -lean_ctor_set(x_73, 1, x_72); -return x_73; +lean_dec(x_8); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_120 = lean_ctor_get(x_115, 0); +lean_inc(x_120); +x_121 = lean_ctor_get(x_115, 1); +lean_inc(x_121); +if (lean_is_exclusive(x_115)) { + lean_ctor_release(x_115, 0); + lean_ctor_release(x_115, 1); + x_122 = x_115; +} else { + lean_dec_ref(x_115); + x_122 = lean_box(0); +} +if (lean_is_scalar(x_122)) { + x_123 = lean_alloc_ctor(1, 2, 0); +} else { + x_123 = x_122; +} +lean_ctor_set(x_123, 0, x_120); +lean_ctor_set(x_123, 1, x_121); +return x_123; } } } else { -lean_object* x_74; lean_object* x_75; lean_object* x_76; -x_74 = lean_ctor_get(x_42, 0); -x_75 = lean_ctor_get(x_42, 1); -lean_inc(x_75); -lean_inc(x_74); -lean_dec(x_42); +uint8_t x_124; +lean_free_object(x_43); +lean_dec(x_47); +lean_dec(x_8); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_124 = !lean_is_exclusive(x_48); +if (x_124 == 0) +{ +return x_48; +} +else +{ +lean_object* x_125; lean_object* x_126; lean_object* x_127; +x_125 = lean_ctor_get(x_48, 0); +x_126 = lean_ctor_get(x_48, 1); +lean_inc(x_126); +lean_inc(x_125); +lean_dec(x_48); +x_127 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_127, 0, x_125); +lean_ctor_set(x_127, 1, x_126); +return x_127; +} +} +} +else +{ +lean_object* x_128; lean_object* x_129; lean_object* x_130; +x_128 = lean_ctor_get(x_43, 0); +x_129 = lean_ctor_get(x_43, 1); +lean_inc(x_129); +lean_inc(x_128); +lean_dec(x_43); +lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); @@ -40840,43 +41083,81 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); -x_76 = l_Lean_Elab_Tactic_renameInaccessibles(x_74, x_38, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_43); -if (lean_obj_tag(x_76) == 0) +x_130 = l_Lean_Elab_Tactic_renameInaccessibles(x_128, x_39, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_44); +if (lean_obj_tag(x_130) == 0) { -lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; -x_77 = lean_ctor_get(x_76, 0); -lean_inc(x_77); -x_78 = lean_ctor_get(x_76, 1); -lean_inc(x_78); -lean_dec(x_76); -x_79 = lean_box(0); -lean_inc(x_77); -x_80 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_80, 0, x_77); -lean_ctor_set(x_80, 1, x_79); -x_81 = l_Lean_Elab_Tactic_setGoals(x_80, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_78); -x_82 = lean_ctor_get(x_81, 1); -lean_inc(x_82); -lean_dec(x_81); -x_83 = lean_box(0); -x_84 = l_Lean_MVarId_setTag(x_77, x_83, x_12, x_13, x_14, x_15, x_82); -x_85 = lean_ctor_get(x_84, 1); -lean_inc(x_85); -lean_dec(x_84); -x_86 = lean_unsigned_to_nat(3u); -x_87 = l_Lean_Elab_Tactic_evalWithAnnotateState___closed__1; -lean_inc(x_1); -x_88 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1), 12, 3); -lean_closure_set(x_88, 0, x_86); -lean_closure_set(x_88, 1, x_87); -lean_closure_set(x_88, 2, x_1); +lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; +x_131 = lean_ctor_get(x_130, 0); +lean_inc(x_131); +x_132 = lean_ctor_get(x_130, 1); +lean_inc(x_132); +lean_dec(x_130); +x_133 = lean_box(0); +lean_inc(x_131); +x_134 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_134, 0, x_131); +lean_ctor_set(x_134, 1, x_133); +x_135 = l_Lean_Elab_Tactic_setGoals(x_134, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_132); +x_136 = lean_ctor_get(x_135, 1); +lean_inc(x_136); +if (lean_is_exclusive(x_135)) { + lean_ctor_release(x_135, 0); + lean_ctor_release(x_135, 1); + x_137 = x_135; +} else { + lean_dec_ref(x_135); + x_137 = lean_box(0); +} +x_138 = lean_box(0); +x_139 = l_Lean_MVarId_setTag(x_131, x_138, x_13, x_14, x_15, x_16, x_136); +x_140 = lean_ctor_get(x_139, 1); +lean_inc(x_140); +if (lean_is_exclusive(x_139)) { + lean_ctor_release(x_139, 0); + lean_ctor_release(x_139, 1); + x_141 = x_139; +} else { + lean_dec_ref(x_139); + x_141 = lean_box(0); +} +lean_inc(x_3); +if (lean_is_scalar(x_141)) { + x_142 = lean_alloc_ctor(1, 2, 0); +} else { + x_142 = x_141; + lean_ctor_set_tag(x_142, 1); +} +lean_ctor_set(x_142, 0, x_3); +lean_ctor_set(x_142, 1, x_133); +lean_inc(x_2); +if (lean_is_scalar(x_137)) { + x_143 = lean_alloc_ctor(1, 2, 0); +} else { + x_143 = x_137; + lean_ctor_set_tag(x_143, 1); +} +lean_ctor_set(x_143, 0, x_2); +lean_ctor_set(x_143, 1, x_142); +x_144 = lean_array_mk(x_143); +x_145 = lean_box(2); +x_146 = l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1___lambda__1___closed__2; +x_147 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_147, 0, x_145); +lean_ctor_set(x_147, 1, x_146); +lean_ctor_set(x_147, 2, x_144); +x_148 = lean_unsigned_to_nat(3u); +x_149 = l_Lean_Elab_Tactic_evalWithAnnotateState___closed__1; lean_inc(x_1); -x_89 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); -lean_closure_set(x_89, 0, x_1); -lean_closure_set(x_89, 1, x_88); -x_90 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_closeUsingOrAdmit), 10, 1); -lean_closure_set(x_90, 0, x_89); +x_150 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1), 12, 3); +lean_closure_set(x_150, 0, x_148); +lean_closure_set(x_150, 1, x_149); +lean_closure_set(x_150, 2, x_1); +x_151 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); +lean_closure_set(x_151, 0, x_147); +lean_closure_set(x_151, 1, x_150); +x_152 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_closeUsingOrAdmit), 10, 1); +lean_closure_set(x_152, 0, x_151); +lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); @@ -40884,31 +41165,31 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); +lean_inc(x_4); lean_inc(x_3); -lean_inc(x_2); -x_91 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalCase___spec__5(x_2, x_3, x_90, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_85); -if (lean_obj_tag(x_91) == 0) +x_153 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalCase___spec__5(x_3, x_4, x_152, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_140); +if (lean_obj_tag(x_153) == 0) { -lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; -x_92 = lean_ctor_get(x_91, 1); -lean_inc(x_92); -lean_dec(x_91); -x_93 = l_Lean_Elab_Tactic_setGoals(x_75, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_92); -x_94 = lean_ctor_get(x_93, 1); -lean_inc(x_94); -lean_dec(x_93); -x_95 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_95, 0, x_7); -x_20 = x_95; -x_21 = x_94; -goto block_28; +lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; +x_154 = lean_ctor_get(x_153, 1); +lean_inc(x_154); +lean_dec(x_153); +x_155 = l_Lean_Elab_Tactic_setGoals(x_129, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_154); +x_156 = lean_ctor_get(x_155, 1); +lean_inc(x_156); +lean_dec(x_155); +x_157 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_157, 0, x_8); +x_21 = x_157; +x_22 = x_156; +goto block_29; } else { -lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; -lean_dec(x_75); -lean_dec(x_7); +lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; +lean_dec(x_129); +lean_dec(x_8); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -40916,37 +41197,38 @@ lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_96 = lean_ctor_get(x_91, 0); -lean_inc(x_96); -x_97 = lean_ctor_get(x_91, 1); -lean_inc(x_97); -if (lean_is_exclusive(x_91)) { - lean_ctor_release(x_91, 0); - lean_ctor_release(x_91, 1); - x_98 = x_91; +x_158 = lean_ctor_get(x_153, 0); +lean_inc(x_158); +x_159 = lean_ctor_get(x_153, 1); +lean_inc(x_159); +if (lean_is_exclusive(x_153)) { + lean_ctor_release(x_153, 0); + lean_ctor_release(x_153, 1); + x_160 = x_153; } else { - lean_dec_ref(x_91); - x_98 = lean_box(0); + lean_dec_ref(x_153); + x_160 = lean_box(0); } -if (lean_is_scalar(x_98)) { - x_99 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_160)) { + x_161 = lean_alloc_ctor(1, 2, 0); } else { - x_99 = x_98; + x_161 = x_160; } -lean_ctor_set(x_99, 0, x_96); -lean_ctor_set(x_99, 1, x_97); -return x_99; +lean_ctor_set(x_161, 0, x_158); +lean_ctor_set(x_161, 1, x_159); +return x_161; } } else { -lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; -lean_dec(x_75); -lean_dec(x_7); +lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; +lean_dec(x_129); +lean_dec(x_8); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -40954,38 +41236,39 @@ lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_100 = lean_ctor_get(x_76, 0); -lean_inc(x_100); -x_101 = lean_ctor_get(x_76, 1); -lean_inc(x_101); -if (lean_is_exclusive(x_76)) { - lean_ctor_release(x_76, 0); - lean_ctor_release(x_76, 1); - x_102 = x_76; +x_162 = lean_ctor_get(x_130, 0); +lean_inc(x_162); +x_163 = lean_ctor_get(x_130, 1); +lean_inc(x_163); +if (lean_is_exclusive(x_130)) { + lean_ctor_release(x_130, 0); + lean_ctor_release(x_130, 1); + x_164 = x_130; } else { - lean_dec_ref(x_76); - x_102 = lean_box(0); + lean_dec_ref(x_130); + x_164 = lean_box(0); } -if (lean_is_scalar(x_102)) { - x_103 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_164)) { + x_165 = lean_alloc_ctor(1, 2, 0); } else { - x_103 = x_102; + x_165 = x_164; } -lean_ctor_set(x_103, 0, x_100); -lean_ctor_set(x_103, 1, x_101); -return x_103; +lean_ctor_set(x_165, 0, x_162); +lean_ctor_set(x_165, 1, x_163); +return x_165; } } } else { -uint8_t x_104; -lean_dec(x_7); -lean_dec(x_38); +uint8_t x_166; +lean_dec(x_8); +lean_dec(x_39); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -40993,63 +41276,64 @@ lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_104 = !lean_is_exclusive(x_41); -if (x_104 == 0) +x_166 = !lean_is_exclusive(x_42); +if (x_166 == 0) { -return x_41; +return x_42; } else { -lean_object* x_105; lean_object* x_106; lean_object* x_107; -x_105 = lean_ctor_get(x_41, 0); -x_106 = lean_ctor_get(x_41, 1); -lean_inc(x_106); -lean_inc(x_105); -lean_dec(x_41); -x_107 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_107, 0, x_105); -lean_ctor_set(x_107, 1, x_106); -return x_107; +lean_object* x_167; lean_object* x_168; lean_object* x_169; +x_167 = lean_ctor_get(x_42, 0); +x_168 = lean_ctor_get(x_42, 1); +lean_inc(x_168); +lean_inc(x_167); +lean_dec(x_42); +x_169 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_169, 0, x_167); +lean_ctor_set(x_169, 1, x_168); +return x_169; } } } else { -lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; -lean_dec(x_7); -x_108 = lean_array_fget(x_29, x_30); -x_109 = lean_unsigned_to_nat(1u); -x_110 = lean_nat_add(x_30, x_109); -lean_dec(x_30); -x_111 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_111, 0, x_29); -lean_ctor_set(x_111, 1, x_110); -lean_ctor_set(x_111, 2, x_31); -x_112 = l___private_Lean_Elab_Tactic_BuiltinTactic_0__Lean_Elab_Tactic_getCaseGoals(x_19, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_112) == 0) +lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; +lean_dec(x_8); +x_170 = lean_array_fget(x_30, x_31); +x_171 = lean_unsigned_to_nat(1u); +x_172 = lean_nat_add(x_31, x_171); +lean_dec(x_31); +x_173 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_173, 0, x_30); +lean_ctor_set(x_173, 1, x_172); +lean_ctor_set(x_173, 2, x_32); +x_174 = l___private_Lean_Elab_Tactic_BuiltinTactic_0__Lean_Elab_Tactic_getCaseGoals(x_20, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +if (lean_obj_tag(x_174) == 0) { -lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; -x_113 = lean_ctor_get(x_112, 0); -lean_inc(x_113); -x_114 = lean_ctor_get(x_112, 1); -lean_inc(x_114); -lean_dec(x_112); -x_115 = lean_ctor_get(x_113, 0); -lean_inc(x_115); -x_116 = lean_ctor_get(x_113, 1); -lean_inc(x_116); -if (lean_is_exclusive(x_113)) { - lean_ctor_release(x_113, 0); - lean_ctor_release(x_113, 1); - x_117 = x_113; +lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; +x_175 = lean_ctor_get(x_174, 0); +lean_inc(x_175); +x_176 = lean_ctor_get(x_174, 1); +lean_inc(x_176); +lean_dec(x_174); +x_177 = lean_ctor_get(x_175, 0); +lean_inc(x_177); +x_178 = lean_ctor_get(x_175, 1); +lean_inc(x_178); +if (lean_is_exclusive(x_175)) { + lean_ctor_release(x_175, 0); + lean_ctor_release(x_175, 1); + x_179 = x_175; } else { - lean_dec_ref(x_113); - x_117 = lean_box(0); + lean_dec_ref(x_175); + x_179 = lean_box(0); } +lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); @@ -41057,48 +41341,86 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); -x_118 = l_Lean_Elab_Tactic_renameInaccessibles(x_115, x_108, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_114); -if (lean_obj_tag(x_118) == 0) +x_180 = l_Lean_Elab_Tactic_renameInaccessibles(x_177, x_170, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_176); +if (lean_obj_tag(x_180) == 0) { -lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; -x_119 = lean_ctor_get(x_118, 0); -lean_inc(x_119); -x_120 = lean_ctor_get(x_118, 1); -lean_inc(x_120); -lean_dec(x_118); -x_121 = lean_box(0); -lean_inc(x_119); -if (lean_is_scalar(x_117)) { - x_122 = lean_alloc_ctor(1, 2, 0); +lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; +x_181 = lean_ctor_get(x_180, 0); +lean_inc(x_181); +x_182 = lean_ctor_get(x_180, 1); +lean_inc(x_182); +lean_dec(x_180); +x_183 = lean_box(0); +lean_inc(x_181); +if (lean_is_scalar(x_179)) { + x_184 = lean_alloc_ctor(1, 2, 0); } else { - x_122 = x_117; - lean_ctor_set_tag(x_122, 1); + x_184 = x_179; + lean_ctor_set_tag(x_184, 1); } -lean_ctor_set(x_122, 0, x_119); -lean_ctor_set(x_122, 1, x_121); -x_123 = l_Lean_Elab_Tactic_setGoals(x_122, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_120); -x_124 = lean_ctor_get(x_123, 1); -lean_inc(x_124); -lean_dec(x_123); -x_125 = lean_box(0); -x_126 = l_Lean_MVarId_setTag(x_119, x_125, x_12, x_13, x_14, x_15, x_124); -x_127 = lean_ctor_get(x_126, 1); -lean_inc(x_127); -lean_dec(x_126); -x_128 = lean_unsigned_to_nat(3u); -x_129 = l_Lean_Elab_Tactic_evalWithAnnotateState___closed__1; -lean_inc(x_1); -x_130 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1), 12, 3); -lean_closure_set(x_130, 0, x_128); -lean_closure_set(x_130, 1, x_129); -lean_closure_set(x_130, 2, x_1); +lean_ctor_set(x_184, 0, x_181); +lean_ctor_set(x_184, 1, x_183); +x_185 = l_Lean_Elab_Tactic_setGoals(x_184, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_182); +x_186 = lean_ctor_get(x_185, 1); +lean_inc(x_186); +if (lean_is_exclusive(x_185)) { + lean_ctor_release(x_185, 0); + lean_ctor_release(x_185, 1); + x_187 = x_185; +} else { + lean_dec_ref(x_185); + x_187 = lean_box(0); +} +x_188 = lean_box(0); +x_189 = l_Lean_MVarId_setTag(x_181, x_188, x_13, x_14, x_15, x_16, x_186); +x_190 = lean_ctor_get(x_189, 1); +lean_inc(x_190); +if (lean_is_exclusive(x_189)) { + lean_ctor_release(x_189, 0); + lean_ctor_release(x_189, 1); + x_191 = x_189; +} else { + lean_dec_ref(x_189); + x_191 = lean_box(0); +} +lean_inc(x_3); +if (lean_is_scalar(x_191)) { + x_192 = lean_alloc_ctor(1, 2, 0); +} else { + x_192 = x_191; + lean_ctor_set_tag(x_192, 1); +} +lean_ctor_set(x_192, 0, x_3); +lean_ctor_set(x_192, 1, x_183); +lean_inc(x_2); +if (lean_is_scalar(x_187)) { + x_193 = lean_alloc_ctor(1, 2, 0); +} else { + x_193 = x_187; + lean_ctor_set_tag(x_193, 1); +} +lean_ctor_set(x_193, 0, x_2); +lean_ctor_set(x_193, 1, x_192); +x_194 = lean_array_mk(x_193); +x_195 = lean_box(2); +x_196 = l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1___lambda__1___closed__2; +x_197 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_197, 0, x_195); +lean_ctor_set(x_197, 1, x_196); +lean_ctor_set(x_197, 2, x_194); +x_198 = lean_unsigned_to_nat(3u); +x_199 = l_Lean_Elab_Tactic_evalWithAnnotateState___closed__1; lean_inc(x_1); -x_131 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); -lean_closure_set(x_131, 0, x_1); -lean_closure_set(x_131, 1, x_130); -x_132 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_closeUsingOrAdmit), 10, 1); -lean_closure_set(x_132, 0, x_131); +x_200 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1), 12, 3); +lean_closure_set(x_200, 0, x_198); +lean_closure_set(x_200, 1, x_199); +lean_closure_set(x_200, 2, x_1); +x_201 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); +lean_closure_set(x_201, 0, x_197); +lean_closure_set(x_201, 1, x_200); +x_202 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_closeUsingOrAdmit), 10, 1); +lean_closure_set(x_202, 0, x_201); +lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); @@ -41106,31 +41428,31 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); +lean_inc(x_4); lean_inc(x_3); -lean_inc(x_2); -x_133 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalCase___spec__5(x_2, x_3, x_132, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_127); -if (lean_obj_tag(x_133) == 0) +x_203 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalCase___spec__5(x_3, x_4, x_202, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_190); +if (lean_obj_tag(x_203) == 0) { -lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; -x_134 = lean_ctor_get(x_133, 1); -lean_inc(x_134); -lean_dec(x_133); -x_135 = l_Lean_Elab_Tactic_setGoals(x_116, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_134); -x_136 = lean_ctor_get(x_135, 1); -lean_inc(x_136); -lean_dec(x_135); -x_137 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_137, 0, x_111); -x_20 = x_137; -x_21 = x_136; -goto block_28; +lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; +x_204 = lean_ctor_get(x_203, 1); +lean_inc(x_204); +lean_dec(x_203); +x_205 = l_Lean_Elab_Tactic_setGoals(x_178, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_204); +x_206 = lean_ctor_get(x_205, 1); +lean_inc(x_206); +lean_dec(x_205); +x_207 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_207, 0, x_173); +x_21 = x_207; +x_22 = x_206; +goto block_29; } else { -lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; -lean_dec(x_116); -lean_dec(x_111); +lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; +lean_dec(x_178); +lean_dec(x_173); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -41138,38 +41460,39 @@ lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_138 = lean_ctor_get(x_133, 0); -lean_inc(x_138); -x_139 = lean_ctor_get(x_133, 1); -lean_inc(x_139); -if (lean_is_exclusive(x_133)) { - lean_ctor_release(x_133, 0); - lean_ctor_release(x_133, 1); - x_140 = x_133; +x_208 = lean_ctor_get(x_203, 0); +lean_inc(x_208); +x_209 = lean_ctor_get(x_203, 1); +lean_inc(x_209); +if (lean_is_exclusive(x_203)) { + lean_ctor_release(x_203, 0); + lean_ctor_release(x_203, 1); + x_210 = x_203; } else { - lean_dec_ref(x_133); - x_140 = lean_box(0); + lean_dec_ref(x_203); + x_210 = lean_box(0); } -if (lean_is_scalar(x_140)) { - x_141 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_210)) { + x_211 = lean_alloc_ctor(1, 2, 0); } else { - x_141 = x_140; + x_211 = x_210; } -lean_ctor_set(x_141, 0, x_138); -lean_ctor_set(x_141, 1, x_139); -return x_141; +lean_ctor_set(x_211, 0, x_208); +lean_ctor_set(x_211, 1, x_209); +return x_211; } } else { -lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; -lean_dec(x_117); -lean_dec(x_116); -lean_dec(x_111); +lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; +lean_dec(x_179); +lean_dec(x_178); +lean_dec(x_173); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -41177,37 +41500,38 @@ lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_142 = lean_ctor_get(x_118, 0); -lean_inc(x_142); -x_143 = lean_ctor_get(x_118, 1); -lean_inc(x_143); -if (lean_is_exclusive(x_118)) { - lean_ctor_release(x_118, 0); - lean_ctor_release(x_118, 1); - x_144 = x_118; +x_212 = lean_ctor_get(x_180, 0); +lean_inc(x_212); +x_213 = lean_ctor_get(x_180, 1); +lean_inc(x_213); +if (lean_is_exclusive(x_180)) { + lean_ctor_release(x_180, 0); + lean_ctor_release(x_180, 1); + x_214 = x_180; } else { - lean_dec_ref(x_118); - x_144 = lean_box(0); + lean_dec_ref(x_180); + x_214 = lean_box(0); } -if (lean_is_scalar(x_144)) { - x_145 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_214)) { + x_215 = lean_alloc_ctor(1, 2, 0); } else { - x_145 = x_144; + x_215 = x_214; } -lean_ctor_set(x_145, 0, x_142); -lean_ctor_set(x_145, 1, x_143); -return x_145; +lean_ctor_set(x_215, 0, x_212); +lean_ctor_set(x_215, 1, x_213); +return x_215; } } else { -lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; -lean_dec(x_111); -lean_dec(x_108); +lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; +lean_dec(x_173); +lean_dec(x_170); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -41215,38 +41539,39 @@ lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_146 = lean_ctor_get(x_112, 0); -lean_inc(x_146); -x_147 = lean_ctor_get(x_112, 1); -lean_inc(x_147); -if (lean_is_exclusive(x_112)) { - lean_ctor_release(x_112, 0); - lean_ctor_release(x_112, 1); - x_148 = x_112; +x_216 = lean_ctor_get(x_174, 0); +lean_inc(x_216); +x_217 = lean_ctor_get(x_174, 1); +lean_inc(x_217); +if (lean_is_exclusive(x_174)) { + lean_ctor_release(x_174, 0); + lean_ctor_release(x_174, 1); + x_218 = x_174; } else { - lean_dec_ref(x_112); - x_148 = lean_box(0); + lean_dec_ref(x_174); + x_218 = lean_box(0); } -if (lean_is_scalar(x_148)) { - x_149 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_218)) { + x_219 = lean_alloc_ctor(1, 2, 0); } else { - x_149 = x_148; + x_219 = x_218; } -lean_ctor_set(x_149, 0, x_146); -lean_ctor_set(x_149, 1, x_147); -return x_149; +lean_ctor_set(x_219, 0, x_216); +lean_ctor_set(x_219, 1, x_217); +return x_219; } } } -block_28: +block_29: { -if (lean_obj_tag(x_20) == 0) +if (lean_obj_tag(x_21) == 0) { -lean_object* x_22; lean_object* x_23; +lean_object* x_23; lean_object* x_24; +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -41254,29 +41579,29 @@ lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_22 = lean_ctor_get(x_20, 0); -lean_inc(x_22); -lean_dec(x_20); -x_23 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_23, 0, x_22); -lean_ctor_set(x_23, 1, x_21); -return x_23; +x_23 = lean_ctor_get(x_21, 0); +lean_inc(x_23); +lean_dec(x_21); +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_23); +lean_ctor_set(x_24, 1, x_22); +return x_24; } else { -lean_object* x_24; size_t x_25; size_t x_26; -x_24 = lean_ctor_get(x_20, 0); -lean_inc(x_24); -lean_dec(x_20); -x_25 = 1; -x_26 = lean_usize_add(x_6, x_25); -x_6 = x_26; -x_7 = x_24; -x_16 = x_21; +lean_object* x_25; size_t x_26; size_t x_27; +x_25 = lean_ctor_get(x_21, 0); +lean_inc(x_25); +lean_dec(x_21); +x_26 = 1; +x_27 = lean_usize_add(x_7, x_26); +x_7 = x_27; +x_8 = x_25; +x_17 = x_22; goto _start; } } @@ -41336,57 +41661,57 @@ return x_11; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalCase___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalCase___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, size_t x_6, size_t x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { _start: { -lean_object* x_17; -x_17 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase___spec__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_17) == 0) +lean_object* x_18; +x_18 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase___spec__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +if (lean_obj_tag(x_18) == 0) { -uint8_t x_18; -x_18 = !lean_is_exclusive(x_17); -if (x_18 == 0) +uint8_t x_19; +x_19 = !lean_is_exclusive(x_18); +if (x_19 == 0) { -lean_object* x_19; lean_object* x_20; -x_19 = lean_ctor_get(x_17, 0); -lean_dec(x_19); -x_20 = lean_box(0); -lean_ctor_set(x_17, 0, x_20); -return x_17; +lean_object* x_20; lean_object* x_21; +x_20 = lean_ctor_get(x_18, 0); +lean_dec(x_20); +x_21 = lean_box(0); +lean_ctor_set(x_18, 0, x_21); +return x_18; } else { -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_17, 1); -lean_inc(x_21); -lean_dec(x_17); -x_22 = lean_box(0); -x_23 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_23, 0, x_22); -lean_ctor_set(x_23, 1, x_21); -return x_23; +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_18, 1); +lean_inc(x_22); +lean_dec(x_18); +x_23 = lean_box(0); +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_23); +lean_ctor_set(x_24, 1, x_22); +return x_24; } } else { -uint8_t x_24; -x_24 = !lean_is_exclusive(x_17); -if (x_24 == 0) +uint8_t x_25; +x_25 = !lean_is_exclusive(x_18); +if (x_25 == 0) { -return x_17; +return x_18; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_17, 0); -x_26 = lean_ctor_get(x_17, 1); +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_18, 0); +x_27 = lean_ctor_get(x_18, 1); +lean_inc(x_27); lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_17); -x_27 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_26); -return x_27; +lean_dec(x_18); +x_28 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +return x_28; } } } @@ -41452,61 +41777,63 @@ return x_13; } else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; -x_14 = lean_unsigned_to_nat(1u); +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; lean_object* x_21; +x_14 = lean_unsigned_to_nat(0u); x_15 = l_Lean_Syntax_getArg(x_1, x_14); -x_16 = l_Lean_Syntax_getArgs(x_15); -lean_dec(x_15); -x_17 = lean_array_get_size(x_16); -x_18 = lean_unsigned_to_nat(0u); -x_19 = lean_nat_dec_lt(x_18, x_17); -if (x_19 == 0) -{ -lean_object* x_50; +x_16 = lean_unsigned_to_nat(1u); +x_17 = l_Lean_Syntax_getArg(x_1, x_16); +x_18 = l_Lean_Syntax_getArgs(x_17); lean_dec(x_17); -lean_dec(x_16); -x_50 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Tactic_evalOpen___spec__3___closed__12; -x_20 = x_50; -goto block_49; +x_19 = lean_array_get_size(x_18); +x_20 = lean_nat_dec_lt(x_14, x_19); +if (x_20 == 0) +{ +lean_object* x_51; +lean_dec(x_19); +lean_dec(x_18); +x_51 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Tactic_evalOpen___spec__3___closed__12; +x_21 = x_51; +goto block_50; } else { -uint8_t x_51; -x_51 = lean_nat_dec_le(x_17, x_17); -if (x_51 == 0) +uint8_t x_52; +x_52 = lean_nat_dec_le(x_19, x_19); +if (x_52 == 0) { -lean_object* x_52; -lean_dec(x_17); -lean_dec(x_16); -x_52 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Tactic_evalOpen___spec__3___closed__12; -x_20 = x_52; -goto block_49; +lean_object* x_53; +lean_dec(x_19); +lean_dec(x_18); +x_53 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Tactic_evalOpen___spec__3___closed__12; +x_21 = x_53; +goto block_50; } else { -size_t x_53; size_t x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; -x_53 = 0; -x_54 = lean_usize_of_nat(x_17); -lean_dec(x_17); -x_55 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Tactic_evalOpen___spec__3___closed__13; -x_56 = l_Array_foldlMUnsafe_fold___at_Lean_Syntax_SepArray_getElems___spec__1(x_16, x_53, x_54, x_55); -lean_dec(x_16); -x_57 = lean_ctor_get(x_56, 1); -lean_inc(x_57); -lean_dec(x_56); -x_20 = x_57; -goto block_49; +size_t x_54; size_t x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; +x_54 = 0; +x_55 = lean_usize_of_nat(x_19); +lean_dec(x_19); +x_56 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Tactic_evalOpen___spec__3___closed__13; +x_57 = l_Array_foldlMUnsafe_fold___at_Lean_Syntax_SepArray_getElems___spec__1(x_18, x_54, x_55, x_56); +lean_dec(x_18); +x_58 = lean_ctor_get(x_57, 1); +lean_inc(x_58); +lean_dec(x_57); +x_21 = x_58; +goto block_50; } } -block_49: +block_50: { -lean_object* x_21; lean_object* x_22; -x_21 = l_Lean_Elab_Tactic_evalCase___closed__3; -x_22 = l_Array_sequenceMap___at_Lean_Elab_Tactic_evalCase___spec__1(x_20, x_21); -lean_dec(x_20); -if (lean_obj_tag(x_22) == 0) +lean_object* x_22; lean_object* x_23; +x_22 = l_Lean_Elab_Tactic_evalCase___closed__3; +x_23 = l_Array_sequenceMap___at_Lean_Elab_Tactic_evalCase___spec__1(x_21, x_22); +lean_dec(x_21); +if (lean_obj_tag(x_23) == 0) { -lean_object* x_23; +lean_object* x_24; +lean_dec(x_15); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -41516,34 +41843,35 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_23 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(x_10); -return x_23; +x_24 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(x_10); +return x_24; } else { -lean_object* x_24; size_t x_25; size_t x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; -x_24 = lean_ctor_get(x_22, 0); -lean_inc(x_24); -lean_dec(x_22); -x_25 = lean_array_size(x_24); -x_26 = 0; -lean_inc(x_24); -x_27 = l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalCase___spec__3(x_25, x_26, x_24); -x_28 = l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalCase___spec__4(x_25, x_26, x_24); -x_29 = lean_unsigned_to_nat(2u); -x_30 = l_Lean_Syntax_getArg(x_1, x_29); -x_31 = lean_unsigned_to_nat(3u); -x_32 = l_Lean_Syntax_getArg(x_1, x_31); -x_33 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_addCheckpoints___spec__1___closed__4; -lean_inc(x_32); -x_34 = l_Lean_Syntax_isOfKind(x_32, x_33); -if (x_34 == 0) +lean_object* x_25; size_t x_26; size_t x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; +x_25 = lean_ctor_get(x_23, 0); +lean_inc(x_25); +lean_dec(x_23); +x_26 = lean_array_size(x_25); +x_27 = 0; +lean_inc(x_25); +x_28 = l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalCase___spec__3(x_26, x_27, x_25); +x_29 = l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalCase___spec__4(x_26, x_27, x_25); +x_30 = lean_unsigned_to_nat(2u); +x_31 = l_Lean_Syntax_getArg(x_1, x_30); +x_32 = lean_unsigned_to_nat(3u); +x_33 = l_Lean_Syntax_getArg(x_1, x_32); +x_34 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_addCheckpoints___spec__1___closed__4; +lean_inc(x_33); +x_35 = l_Lean_Syntax_isOfKind(x_33, x_34); +if (x_35 == 0) { -lean_object* x_35; -lean_dec(x_32); -lean_dec(x_30); +lean_object* x_36; +lean_dec(x_33); +lean_dec(x_31); +lean_dec(x_29); lean_dec(x_28); -lean_dec(x_27); +lean_dec(x_15); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -41553,24 +41881,25 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_35 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(x_10); -return x_35; +x_36 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(x_10); +return x_36; } else { -lean_object* x_36; lean_object* x_37; uint8_t x_38; -x_36 = l_Lean_Syntax_getArg(x_32, x_18); -lean_dec(x_32); -x_37 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_addCheckpoints___spec__1___closed__6; -lean_inc(x_36); -x_38 = l_Lean_Syntax_isOfKind(x_36, x_37); -if (x_38 == 0) +lean_object* x_37; lean_object* x_38; uint8_t x_39; +x_37 = l_Lean_Syntax_getArg(x_33, x_14); +lean_dec(x_33); +x_38 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_addCheckpoints___spec__1___closed__6; +lean_inc(x_37); +x_39 = l_Lean_Syntax_isOfKind(x_37, x_38); +if (x_39 == 0) { -lean_object* x_39; -lean_dec(x_36); -lean_dec(x_30); +lean_object* x_40; +lean_dec(x_37); +lean_dec(x_31); +lean_dec(x_29); lean_dec(x_28); -lean_dec(x_27); +lean_dec(x_15); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -41580,30 +41909,31 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_39 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(x_10); -return x_39; +x_40 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(x_10); +return x_40; } else { -lean_object* x_40; uint8_t x_41; lean_object* x_42; lean_object* x_43; size_t x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; -x_40 = lean_array_get_size(x_28); -x_41 = lean_nat_dec_lt(x_14, x_40); -lean_dec(x_40); -x_42 = lean_array_get_size(x_27); -x_43 = l_Array_toSubarray___rarg(x_27, x_18, x_42); -x_44 = lean_array_size(x_28); -x_45 = lean_box_usize(x_44); -x_46 = l_Lean_Elab_Tactic_evalCase___boxed__const__1; -x_47 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalCase___lambda__2___boxed), 16, 7); -lean_closure_set(x_47, 0, x_1); -lean_closure_set(x_47, 1, x_30); -lean_closure_set(x_47, 2, x_36); -lean_closure_set(x_47, 3, x_28); -lean_closure_set(x_47, 4, x_45); -lean_closure_set(x_47, 5, x_46); -lean_closure_set(x_47, 6, x_43); -x_48 = l_Lean_Elab_Term_withoutTacticIncrementality___at_Lean_Elab_Tactic_evalTactic_eval___spec__3(x_41, x_47, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_48; +lean_object* x_41; uint8_t x_42; lean_object* x_43; lean_object* x_44; size_t x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_41 = lean_array_get_size(x_29); +x_42 = lean_nat_dec_lt(x_16, x_41); +lean_dec(x_41); +x_43 = lean_array_get_size(x_28); +x_44 = l_Array_toSubarray___rarg(x_28, x_14, x_43); +x_45 = lean_array_size(x_29); +x_46 = lean_box_usize(x_45); +x_47 = l_Lean_Elab_Tactic_evalCase___boxed__const__1; +x_48 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalCase___lambda__2___boxed), 17, 8); +lean_closure_set(x_48, 0, x_1); +lean_closure_set(x_48, 1, x_15); +lean_closure_set(x_48, 2, x_31); +lean_closure_set(x_48, 3, x_37); +lean_closure_set(x_48, 4, x_29); +lean_closure_set(x_48, 5, x_46); +lean_closure_set(x_48, 6, x_47); +lean_closure_set(x_48, 7, x_44); +x_49 = l_Lean_Elab_Term_withoutTacticIncrementality___at_Lean_Elab_Tactic_evalTactic_eval___spec__3(x_42, x_48, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_49; } } } @@ -41653,30 +41983,64 @@ x_6 = l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalCase___spec__4(x_4, x_5, return x_6; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase___spec__6___boxed(lean_object** _args) { +lean_object* x_1 = _args[0]; +lean_object* x_2 = _args[1]; +lean_object* x_3 = _args[2]; +lean_object* x_4 = _args[3]; +lean_object* x_5 = _args[4]; +lean_object* x_6 = _args[5]; +lean_object* x_7 = _args[6]; +lean_object* x_8 = _args[7]; +lean_object* x_9 = _args[8]; +lean_object* x_10 = _args[9]; +lean_object* x_11 = _args[10]; +lean_object* x_12 = _args[11]; +lean_object* x_13 = _args[12]; +lean_object* x_14 = _args[13]; +lean_object* x_15 = _args[14]; +lean_object* x_16 = _args[15]; +lean_object* x_17 = _args[16]; _start: { -size_t x_17; size_t x_18; lean_object* x_19; -x_17 = lean_unbox_usize(x_5); -lean_dec(x_5); +size_t x_18; size_t x_19; lean_object* x_20; x_18 = lean_unbox_usize(x_6); lean_dec(x_6); -x_19 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase___spec__6(x_1, x_2, x_3, x_4, x_17, x_18, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_4); -return x_19; +x_19 = lean_unbox_usize(x_7); +lean_dec(x_7); +x_20 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase___spec__6(x_1, x_2, x_3, x_4, x_5, x_18, x_19, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +lean_dec(x_5); +return x_20; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalCase___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalCase___lambda__2___boxed(lean_object** _args) { +lean_object* x_1 = _args[0]; +lean_object* x_2 = _args[1]; +lean_object* x_3 = _args[2]; +lean_object* x_4 = _args[3]; +lean_object* x_5 = _args[4]; +lean_object* x_6 = _args[5]; +lean_object* x_7 = _args[6]; +lean_object* x_8 = _args[7]; +lean_object* x_9 = _args[8]; +lean_object* x_10 = _args[9]; +lean_object* x_11 = _args[10]; +lean_object* x_12 = _args[11]; +lean_object* x_13 = _args[12]; +lean_object* x_14 = _args[13]; +lean_object* x_15 = _args[14]; +lean_object* x_16 = _args[15]; +lean_object* x_17 = _args[16]; _start: { -size_t x_17; size_t x_18; lean_object* x_19; -x_17 = lean_unbox_usize(x_5); -lean_dec(x_5); +size_t x_18; size_t x_19; lean_object* x_20; x_18 = lean_unbox_usize(x_6); lean_dec(x_6); -x_19 = l_Lean_Elab_Tactic_evalCase___lambda__2(x_1, x_2, x_3, x_4, x_17, x_18, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_4); -return x_19; +x_19 = lean_unbox_usize(x_7); +lean_dec(x_7); +x_20 = l_Lean_Elab_Tactic_evalCase___lambda__2(x_1, x_2, x_3, x_4, x_5, x_18, x_19, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +lean_dec(x_5); +return x_20; } } static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalCase__1___closed__1() { @@ -41868,14 +42232,15 @@ return x_24; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, size_t x_6, size_t x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { _start: { -uint8_t x_17; -x_17 = lean_usize_dec_lt(x_6, x_5); -if (x_17 == 0) +uint8_t x_18; +x_18 = lean_usize_dec_lt(x_7, x_6); +if (x_18 == 0) { -lean_object* x_18; +lean_object* x_19; +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -41883,79 +42248,80 @@ lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_7); -lean_ctor_set(x_18, 1, x_16); -return x_18; +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_8); +lean_ctor_set(x_19, 1, x_17); +return x_19; } else { -lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_29; -x_19 = lean_array_uget(x_4, x_6); -x_29 = !lean_is_exclusive(x_7); -if (x_29 == 0) +lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_30; +x_20 = lean_array_uget(x_5, x_7); +x_30 = !lean_is_exclusive(x_8); +if (x_30 == 0) { -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; -x_30 = lean_ctor_get(x_7, 0); -x_31 = lean_ctor_get(x_7, 1); -x_32 = lean_ctor_get(x_30, 0); -lean_inc(x_32); -x_33 = lean_ctor_get(x_30, 1); +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; +x_31 = lean_ctor_get(x_8, 0); +x_32 = lean_ctor_get(x_8, 1); +x_33 = lean_ctor_get(x_31, 0); lean_inc(x_33); -x_34 = lean_ctor_get(x_30, 2); +x_34 = lean_ctor_get(x_31, 1); lean_inc(x_34); -x_35 = lean_nat_dec_lt(x_33, x_34); -if (x_35 == 0) +x_35 = lean_ctor_get(x_31, 2); +lean_inc(x_35); +x_36 = lean_nat_dec_lt(x_34, x_35); +if (x_36 == 0) { -lean_object* x_36; +lean_object* x_37; +lean_dec(x_35); lean_dec(x_34); lean_dec(x_33); -lean_dec(x_32); -lean_dec(x_19); -x_36 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_36, 0, x_7); -x_20 = x_36; -x_21 = x_16; -goto block_28; +lean_dec(x_20); +x_37 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_37, 0, x_8); +x_21 = x_37; +x_22 = x_17; +goto block_29; } else { -uint8_t x_37; -lean_free_object(x_7); -x_37 = !lean_is_exclusive(x_30); -if (x_37 == 0) +uint8_t x_38; +lean_free_object(x_8); +x_38 = !lean_is_exclusive(x_31); +if (x_38 == 0) { -lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_38 = lean_ctor_get(x_30, 2); -lean_dec(x_38); -x_39 = lean_ctor_get(x_30, 1); +lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_39 = lean_ctor_get(x_31, 2); lean_dec(x_39); -x_40 = lean_ctor_get(x_30, 0); +x_40 = lean_ctor_get(x_31, 1); lean_dec(x_40); -x_41 = lean_array_fget(x_32, x_33); -x_42 = lean_unsigned_to_nat(1u); -x_43 = lean_nat_add(x_33, x_42); -lean_dec(x_33); -lean_ctor_set(x_30, 1, x_43); -x_44 = l___private_Lean_Elab_Tactic_BuiltinTactic_0__Lean_Elab_Tactic_getCaseGoals(x_19, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_44) == 0) +x_41 = lean_ctor_get(x_31, 0); +lean_dec(x_41); +x_42 = lean_array_fget(x_33, x_34); +x_43 = lean_unsigned_to_nat(1u); +x_44 = lean_nat_add(x_34, x_43); +lean_dec(x_34); +lean_ctor_set(x_31, 1, x_44); +x_45 = l___private_Lean_Elab_Tactic_BuiltinTactic_0__Lean_Elab_Tactic_getCaseGoals(x_20, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +if (lean_obj_tag(x_45) == 0) { -lean_object* x_45; lean_object* x_46; uint8_t x_47; -x_45 = lean_ctor_get(x_44, 0); -lean_inc(x_45); -x_46 = lean_ctor_get(x_44, 1); +lean_object* x_46; lean_object* x_47; uint8_t x_48; +x_46 = lean_ctor_get(x_45, 0); lean_inc(x_46); -lean_dec(x_44); -x_47 = !lean_is_exclusive(x_45); -if (x_47 == 0) +x_47 = lean_ctor_get(x_45, 1); +lean_inc(x_47); +lean_dec(x_45); +x_48 = !lean_is_exclusive(x_46); +if (x_48 == 0) { -lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_ctor_get(x_45, 0); -x_49 = lean_ctor_get(x_45, 1); +lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_49 = lean_ctor_get(x_46, 0); +x_50 = lean_ctor_get(x_46, 1); +lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); @@ -41963,37 +42329,60 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); -x_50 = l_Lean_Elab_Tactic_renameInaccessibles(x_48, x_41, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_46); -if (lean_obj_tag(x_50) == 0) +x_51 = l_Lean_Elab_Tactic_renameInaccessibles(x_49, x_42, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_47); +if (lean_obj_tag(x_51) == 0) { -lean_object* x_51; lean_object* x_52; lean_object* x_53; -x_51 = lean_ctor_get(x_50, 0); -lean_inc(x_51); -x_52 = lean_ctor_get(x_50, 1); +lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_52 = lean_ctor_get(x_51, 0); lean_inc(x_52); -lean_dec(x_50); -lean_inc(x_51); -x_53 = l_Lean_MVarId_getTag(x_51, x_12, x_13, x_14, x_15, x_52); -if (lean_obj_tag(x_53) == 0) +x_53 = lean_ctor_get(x_51, 1); +lean_inc(x_53); +lean_dec(x_51); +lean_inc(x_52); +x_54 = l_Lean_MVarId_getTag(x_52, x_13, x_14, x_15, x_16, x_53); +if (lean_obj_tag(x_54) == 0) { -lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; -x_54 = lean_ctor_get(x_53, 0); -lean_inc(x_54); -x_55 = lean_ctor_get(x_53, 1); +lean_object* x_55; lean_object* x_56; lean_object* x_57; uint8_t x_58; +x_55 = lean_ctor_get(x_54, 0); lean_inc(x_55); -lean_dec(x_53); -lean_inc(x_3); -lean_ctor_set_tag(x_45, 1); -lean_ctor_set(x_45, 1, x_3); -lean_ctor_set(x_45, 0, x_51); -x_56 = l_Lean_Elab_Tactic_setGoals(x_45, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_55); -x_57 = lean_ctor_get(x_56, 1); -lean_inc(x_57); -lean_dec(x_56); +x_56 = lean_ctor_get(x_54, 1); +lean_inc(x_56); +lean_dec(x_54); +lean_inc(x_4); +lean_ctor_set_tag(x_46, 1); +lean_ctor_set(x_46, 1, x_4); +lean_ctor_set(x_46, 0, x_52); +x_57 = l_Lean_Elab_Tactic_setGoals(x_46, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_56); +x_58 = !lean_is_exclusive(x_57); +if (x_58 == 0) +{ +lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; +x_59 = lean_ctor_get(x_57, 1); +x_60 = lean_ctor_get(x_57, 0); +lean_dec(x_60); +x_61 = lean_box(0); lean_inc(x_2); -x_58 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalTactic), 10, 1); -lean_closure_set(x_58, 0, x_2); +lean_ctor_set_tag(x_57, 1); +lean_ctor_set(x_57, 1, x_61); +lean_ctor_set(x_57, 0, x_2); +lean_inc(x_1); +x_62 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_62, 0, x_1); +lean_ctor_set(x_62, 1, x_57); +x_63 = lean_array_mk(x_62); +x_64 = lean_box(2); +x_65 = l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1___lambda__1___closed__2; +x_66 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_66, 0, x_64); +lean_ctor_set(x_66, 1, x_65); +lean_ctor_set(x_66, 2, x_63); +lean_inc(x_3); +x_67 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalTactic), 10, 1); +lean_closure_set(x_67, 0, x_3); +x_68 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); +lean_closure_set(x_68, 0, x_66); +lean_closure_set(x_68, 1, x_67); +lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); @@ -42001,172 +42390,95 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); +lean_inc(x_3); lean_inc(x_2); -lean_inc(x_1); -x_59 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalCase___spec__5(x_1, x_2, x_58, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_57); -if (lean_obj_tag(x_59) == 0) -{ -lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_60 = lean_ctor_get(x_59, 1); -lean_inc(x_60); -lean_dec(x_59); -x_61 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_60); -x_62 = lean_ctor_get(x_61, 0); -lean_inc(x_62); -if (lean_obj_tag(x_62) == 0) -{ -lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; -lean_dec(x_54); -x_63 = lean_ctor_get(x_61, 1); -lean_inc(x_63); -lean_dec(x_61); -x_64 = lean_box(0); -x_65 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_62, x_49, x_30, x_31, x_64, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_63); -x_66 = lean_ctor_get(x_65, 0); -lean_inc(x_66); -x_67 = lean_ctor_get(x_65, 1); -lean_inc(x_67); -lean_dec(x_65); -x_20 = x_66; -x_21 = x_67; -goto block_28; -} -else -{ -lean_object* x_68; -x_68 = lean_ctor_get(x_62, 1); -lean_inc(x_68); -if (lean_obj_tag(x_68) == 0) +x_69 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalCase___spec__5(x_2, x_3, x_68, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_59); +if (lean_obj_tag(x_69) == 0) { -lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; -x_69 = lean_ctor_get(x_61, 1); -lean_inc(x_69); -lean_dec(x_61); -x_70 = lean_ctor_get(x_62, 0); +lean_object* x_70; lean_object* x_71; lean_object* x_72; +x_70 = lean_ctor_get(x_69, 1); lean_inc(x_70); -x_71 = l_Lean_MVarId_setTag(x_70, x_54, x_12, x_13, x_14, x_15, x_69); +lean_dec(x_69); +x_71 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_70); x_72 = lean_ctor_get(x_71, 0); lean_inc(x_72); +if (lean_obj_tag(x_72) == 0) +{ +lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; +lean_dec(x_55); x_73 = lean_ctor_get(x_71, 1); lean_inc(x_73); lean_dec(x_71); -x_74 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_62, x_49, x_30, x_31, x_72, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_73); -lean_dec(x_72); -x_75 = lean_ctor_get(x_74, 0); -lean_inc(x_75); -x_76 = lean_ctor_get(x_74, 1); +x_74 = lean_box(0); +x_75 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_72, x_50, x_31, x_32, x_74, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_73); +x_76 = lean_ctor_get(x_75, 0); lean_inc(x_76); -lean_dec(x_74); -x_20 = x_75; -x_21 = x_76; -goto block_28; -} -else -{ -lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; -lean_dec(x_68); -lean_dec(x_54); -x_77 = lean_ctor_get(x_61, 1); +x_77 = lean_ctor_get(x_75, 1); lean_inc(x_77); -lean_dec(x_61); -x_78 = lean_box(0); -x_79 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_62, x_49, x_30, x_31, x_78, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_77); -x_80 = lean_ctor_get(x_79, 0); -lean_inc(x_80); -x_81 = lean_ctor_get(x_79, 1); -lean_inc(x_81); -lean_dec(x_79); -x_20 = x_80; -x_21 = x_81; -goto block_28; -} -} +lean_dec(x_75); +x_21 = x_76; +x_22 = x_77; +goto block_29; } else { -uint8_t x_82; -lean_dec(x_54); -lean_dec(x_49); -lean_dec(x_30); -lean_dec(x_31); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_82 = !lean_is_exclusive(x_59); -if (x_82 == 0) -{ -return x_59; -} -else +lean_object* x_78; +x_78 = lean_ctor_get(x_72, 1); +lean_inc(x_78); +if (lean_obj_tag(x_78) == 0) { -lean_object* x_83; lean_object* x_84; lean_object* x_85; -x_83 = lean_ctor_get(x_59, 0); -x_84 = lean_ctor_get(x_59, 1); -lean_inc(x_84); +lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; +x_79 = lean_ctor_get(x_71, 1); +lean_inc(x_79); +lean_dec(x_71); +x_80 = lean_ctor_get(x_72, 0); +lean_inc(x_80); +x_81 = l_Lean_MVarId_setTag(x_80, x_55, x_13, x_14, x_15, x_16, x_79); +x_82 = lean_ctor_get(x_81, 0); +lean_inc(x_82); +x_83 = lean_ctor_get(x_81, 1); lean_inc(x_83); -lean_dec(x_59); -x_85 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_85, 0, x_83); -lean_ctor_set(x_85, 1, x_84); -return x_85; -} -} -} -else -{ -uint8_t x_86; -lean_dec(x_51); -lean_free_object(x_45); -lean_dec(x_49); -lean_dec(x_30); -lean_dec(x_31); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_86 = !lean_is_exclusive(x_53); -if (x_86 == 0) -{ -return x_53; +lean_dec(x_81); +x_84 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_72, x_50, x_31, x_32, x_82, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_83); +lean_dec(x_82); +x_85 = lean_ctor_get(x_84, 0); +lean_inc(x_85); +x_86 = lean_ctor_get(x_84, 1); +lean_inc(x_86); +lean_dec(x_84); +x_21 = x_85; +x_22 = x_86; +goto block_29; } else { -lean_object* x_87; lean_object* x_88; lean_object* x_89; -x_87 = lean_ctor_get(x_53, 0); -x_88 = lean_ctor_get(x_53, 1); -lean_inc(x_88); +lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; +lean_dec(x_78); +lean_dec(x_55); +x_87 = lean_ctor_get(x_71, 1); lean_inc(x_87); -lean_dec(x_53); -x_89 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_89, 0, x_87); -lean_ctor_set(x_89, 1, x_88); -return x_89; +lean_dec(x_71); +x_88 = lean_box(0); +x_89 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_72, x_50, x_31, x_32, x_88, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_87); +x_90 = lean_ctor_get(x_89, 0); +lean_inc(x_90); +x_91 = lean_ctor_get(x_89, 1); +lean_inc(x_91); +lean_dec(x_89); +x_21 = x_90; +x_22 = x_91; +goto block_29; } } } else { -uint8_t x_90; -lean_free_object(x_45); -lean_dec(x_49); -lean_dec(x_30); +uint8_t x_92; +lean_dec(x_55); +lean_dec(x_50); lean_dec(x_31); +lean_dec(x_32); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -42174,76 +42486,59 @@ lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_90 = !lean_is_exclusive(x_50); -if (x_90 == 0) +x_92 = !lean_is_exclusive(x_69); +if (x_92 == 0) { -return x_50; +return x_69; } else { -lean_object* x_91; lean_object* x_92; lean_object* x_93; -x_91 = lean_ctor_get(x_50, 0); -x_92 = lean_ctor_get(x_50, 1); -lean_inc(x_92); -lean_inc(x_91); -lean_dec(x_50); -x_93 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_93, 0, x_91); -lean_ctor_set(x_93, 1, x_92); -return x_93; +lean_object* x_93; lean_object* x_94; lean_object* x_95; +x_93 = lean_ctor_get(x_69, 0); +x_94 = lean_ctor_get(x_69, 1); +lean_inc(x_94); +lean_inc(x_93); +lean_dec(x_69); +x_95 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_95, 0, x_93); +lean_ctor_set(x_95, 1, x_94); +return x_95; } } } else { -lean_object* x_94; lean_object* x_95; lean_object* x_96; -x_94 = lean_ctor_get(x_45, 0); -x_95 = lean_ctor_get(x_45, 1); -lean_inc(x_95); -lean_inc(x_94); -lean_dec(x_45); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -x_96 = l_Lean_Elab_Tactic_renameInaccessibles(x_94, x_41, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_46); -if (lean_obj_tag(x_96) == 0) -{ -lean_object* x_97; lean_object* x_98; lean_object* x_99; -x_97 = lean_ctor_get(x_96, 0); -lean_inc(x_97); -x_98 = lean_ctor_get(x_96, 1); -lean_inc(x_98); -lean_dec(x_96); -lean_inc(x_97); -x_99 = l_Lean_MVarId_getTag(x_97, x_12, x_13, x_14, x_15, x_98); -if (lean_obj_tag(x_99) == 0) -{ -lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; -x_100 = lean_ctor_get(x_99, 0); -lean_inc(x_100); -x_101 = lean_ctor_get(x_99, 1); -lean_inc(x_101); -lean_dec(x_99); -lean_inc(x_3); -x_102 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_102, 0, x_97); -lean_ctor_set(x_102, 1, x_3); -x_103 = l_Lean_Elab_Tactic_setGoals(x_102, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_101); -x_104 = lean_ctor_get(x_103, 1); -lean_inc(x_104); -lean_dec(x_103); +lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; +x_96 = lean_ctor_get(x_57, 1); +lean_inc(x_96); +lean_dec(x_57); +x_97 = lean_box(0); lean_inc(x_2); -x_105 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalTactic), 10, 1); -lean_closure_set(x_105, 0, x_2); +x_98 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_98, 0, x_2); +lean_ctor_set(x_98, 1, x_97); +lean_inc(x_1); +x_99 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_99, 0, x_1); +lean_ctor_set(x_99, 1, x_98); +x_100 = lean_array_mk(x_99); +x_101 = lean_box(2); +x_102 = l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1___lambda__1___closed__2; +x_103 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_103, 0, x_101); +lean_ctor_set(x_103, 1, x_102); +lean_ctor_set(x_103, 2, x_100); +lean_inc(x_3); +x_104 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalTactic), 10, 1); +lean_closure_set(x_104, 0, x_3); +x_105 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); +lean_closure_set(x_105, 0, x_103); +lean_closure_set(x_105, 1, x_104); +lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); @@ -42251,36 +42546,35 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); +lean_inc(x_3); lean_inc(x_2); -lean_inc(x_1); -x_106 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalCase___spec__5(x_1, x_2, x_105, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_104); +x_106 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalCase___spec__5(x_2, x_3, x_105, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_96); if (lean_obj_tag(x_106) == 0) { lean_object* x_107; lean_object* x_108; lean_object* x_109; x_107 = lean_ctor_get(x_106, 1); lean_inc(x_107); lean_dec(x_106); -x_108 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_107); +x_108 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_107); x_109 = lean_ctor_get(x_108, 0); lean_inc(x_109); if (lean_obj_tag(x_109) == 0) { lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; -lean_dec(x_100); +lean_dec(x_55); x_110 = lean_ctor_get(x_108, 1); lean_inc(x_110); lean_dec(x_108); x_111 = lean_box(0); -x_112 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_109, x_95, x_30, x_31, x_111, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_110); +x_112 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_109, x_50, x_31, x_32, x_111, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_110); x_113 = lean_ctor_get(x_112, 0); lean_inc(x_113); x_114 = lean_ctor_get(x_112, 1); lean_inc(x_114); lean_dec(x_112); -x_20 = x_113; -x_21 = x_114; -goto block_28; +x_21 = x_113; +x_22 = x_114; +goto block_29; } else { @@ -42295,51 +42589,52 @@ lean_inc(x_116); lean_dec(x_108); x_117 = lean_ctor_get(x_109, 0); lean_inc(x_117); -x_118 = l_Lean_MVarId_setTag(x_117, x_100, x_12, x_13, x_14, x_15, x_116); +x_118 = l_Lean_MVarId_setTag(x_117, x_55, x_13, x_14, x_15, x_16, x_116); x_119 = lean_ctor_get(x_118, 0); lean_inc(x_119); x_120 = lean_ctor_get(x_118, 1); lean_inc(x_120); lean_dec(x_118); -x_121 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_109, x_95, x_30, x_31, x_119, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_120); +x_121 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_109, x_50, x_31, x_32, x_119, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_120); lean_dec(x_119); x_122 = lean_ctor_get(x_121, 0); lean_inc(x_122); x_123 = lean_ctor_get(x_121, 1); lean_inc(x_123); lean_dec(x_121); -x_20 = x_122; -x_21 = x_123; -goto block_28; +x_21 = x_122; +x_22 = x_123; +goto block_29; } else { lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_dec(x_115); -lean_dec(x_100); +lean_dec(x_55); x_124 = lean_ctor_get(x_108, 1); lean_inc(x_124); lean_dec(x_108); x_125 = lean_box(0); -x_126 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_109, x_95, x_30, x_31, x_125, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_124); +x_126 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_109, x_50, x_31, x_32, x_125, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_124); x_127 = lean_ctor_get(x_126, 0); lean_inc(x_127); x_128 = lean_ctor_get(x_126, 1); lean_inc(x_128); lean_dec(x_126); -x_20 = x_127; -x_21 = x_128; -goto block_28; +x_21 = x_127; +x_22 = x_128; +goto block_29; } } } else { lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; -lean_dec(x_100); -lean_dec(x_95); -lean_dec(x_30); +lean_dec(x_55); +lean_dec(x_50); lean_dec(x_31); +lean_dec(x_32); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -42347,7 +42642,7 @@ lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); @@ -42373,13 +42668,16 @@ lean_ctor_set(x_132, 1, x_130); return x_132; } } +} else { -lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; -lean_dec(x_97); -lean_dec(x_95); -lean_dec(x_30); +uint8_t x_133; +lean_dec(x_52); +lean_free_object(x_46); +lean_dec(x_50); lean_dec(x_31); +lean_dec(x_32); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -42387,38 +42685,324 @@ lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_133 = lean_ctor_get(x_99, 0); -lean_inc(x_133); -x_134 = lean_ctor_get(x_99, 1); +x_133 = !lean_is_exclusive(x_54); +if (x_133 == 0) +{ +return x_54; +} +else +{ +lean_object* x_134; lean_object* x_135; lean_object* x_136; +x_134 = lean_ctor_get(x_54, 0); +x_135 = lean_ctor_get(x_54, 1); +lean_inc(x_135); lean_inc(x_134); -if (lean_is_exclusive(x_99)) { - lean_ctor_release(x_99, 0); - lean_ctor_release(x_99, 1); - x_135 = x_99; +lean_dec(x_54); +x_136 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_136, 0, x_134); +lean_ctor_set(x_136, 1, x_135); +return x_136; +} +} +} +else +{ +uint8_t x_137; +lean_free_object(x_46); +lean_dec(x_50); +lean_dec(x_31); +lean_dec(x_32); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_137 = !lean_is_exclusive(x_51); +if (x_137 == 0) +{ +return x_51; +} +else +{ +lean_object* x_138; lean_object* x_139; lean_object* x_140; +x_138 = lean_ctor_get(x_51, 0); +x_139 = lean_ctor_get(x_51, 1); +lean_inc(x_139); +lean_inc(x_138); +lean_dec(x_51); +x_140 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_140, 0, x_138); +lean_ctor_set(x_140, 1, x_139); +return x_140; +} +} +} +else +{ +lean_object* x_141; lean_object* x_142; lean_object* x_143; +x_141 = lean_ctor_get(x_46, 0); +x_142 = lean_ctor_get(x_46, 1); +lean_inc(x_142); +lean_inc(x_141); +lean_dec(x_46); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +x_143 = l_Lean_Elab_Tactic_renameInaccessibles(x_141, x_42, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_47); +if (lean_obj_tag(x_143) == 0) +{ +lean_object* x_144; lean_object* x_145; lean_object* x_146; +x_144 = lean_ctor_get(x_143, 0); +lean_inc(x_144); +x_145 = lean_ctor_get(x_143, 1); +lean_inc(x_145); +lean_dec(x_143); +lean_inc(x_144); +x_146 = l_Lean_MVarId_getTag(x_144, x_13, x_14, x_15, x_16, x_145); +if (lean_obj_tag(x_146) == 0) +{ +lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; +x_147 = lean_ctor_get(x_146, 0); +lean_inc(x_147); +x_148 = lean_ctor_get(x_146, 1); +lean_inc(x_148); +lean_dec(x_146); +lean_inc(x_4); +x_149 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_149, 0, x_144); +lean_ctor_set(x_149, 1, x_4); +x_150 = l_Lean_Elab_Tactic_setGoals(x_149, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_148); +x_151 = lean_ctor_get(x_150, 1); +lean_inc(x_151); +if (lean_is_exclusive(x_150)) { + lean_ctor_release(x_150, 0); + lean_ctor_release(x_150, 1); + x_152 = x_150; } else { - lean_dec_ref(x_99); - x_135 = lean_box(0); + lean_dec_ref(x_150); + x_152 = lean_box(0); +} +x_153 = lean_box(0); +lean_inc(x_2); +if (lean_is_scalar(x_152)) { + x_154 = lean_alloc_ctor(1, 2, 0); +} else { + x_154 = x_152; + lean_ctor_set_tag(x_154, 1); +} +lean_ctor_set(x_154, 0, x_2); +lean_ctor_set(x_154, 1, x_153); +lean_inc(x_1); +x_155 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_155, 0, x_1); +lean_ctor_set(x_155, 1, x_154); +x_156 = lean_array_mk(x_155); +x_157 = lean_box(2); +x_158 = l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1___lambda__1___closed__2; +x_159 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_159, 0, x_157); +lean_ctor_set(x_159, 1, x_158); +lean_ctor_set(x_159, 2, x_156); +lean_inc(x_3); +x_160 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalTactic), 10, 1); +lean_closure_set(x_160, 0, x_3); +x_161 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); +lean_closure_set(x_161, 0, x_159); +lean_closure_set(x_161, 1, x_160); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_3); +lean_inc(x_2); +x_162 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalCase___spec__5(x_2, x_3, x_161, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_151); +if (lean_obj_tag(x_162) == 0) +{ +lean_object* x_163; lean_object* x_164; lean_object* x_165; +x_163 = lean_ctor_get(x_162, 1); +lean_inc(x_163); +lean_dec(x_162); +x_164 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_163); +x_165 = lean_ctor_get(x_164, 0); +lean_inc(x_165); +if (lean_obj_tag(x_165) == 0) +{ +lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; +lean_dec(x_147); +x_166 = lean_ctor_get(x_164, 1); +lean_inc(x_166); +lean_dec(x_164); +x_167 = lean_box(0); +x_168 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_165, x_142, x_31, x_32, x_167, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_166); +x_169 = lean_ctor_get(x_168, 0); +lean_inc(x_169); +x_170 = lean_ctor_get(x_168, 1); +lean_inc(x_170); +lean_dec(x_168); +x_21 = x_169; +x_22 = x_170; +goto block_29; +} +else +{ +lean_object* x_171; +x_171 = lean_ctor_get(x_165, 1); +lean_inc(x_171); +if (lean_obj_tag(x_171) == 0) +{ +lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; +x_172 = lean_ctor_get(x_164, 1); +lean_inc(x_172); +lean_dec(x_164); +x_173 = lean_ctor_get(x_165, 0); +lean_inc(x_173); +x_174 = l_Lean_MVarId_setTag(x_173, x_147, x_13, x_14, x_15, x_16, x_172); +x_175 = lean_ctor_get(x_174, 0); +lean_inc(x_175); +x_176 = lean_ctor_get(x_174, 1); +lean_inc(x_176); +lean_dec(x_174); +x_177 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_165, x_142, x_31, x_32, x_175, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_176); +lean_dec(x_175); +x_178 = lean_ctor_get(x_177, 0); +lean_inc(x_178); +x_179 = lean_ctor_get(x_177, 1); +lean_inc(x_179); +lean_dec(x_177); +x_21 = x_178; +x_22 = x_179; +goto block_29; +} +else +{ +lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; +lean_dec(x_171); +lean_dec(x_147); +x_180 = lean_ctor_get(x_164, 1); +lean_inc(x_180); +lean_dec(x_164); +x_181 = lean_box(0); +x_182 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_165, x_142, x_31, x_32, x_181, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_180); +x_183 = lean_ctor_get(x_182, 0); +lean_inc(x_183); +x_184 = lean_ctor_get(x_182, 1); +lean_inc(x_184); +lean_dec(x_182); +x_21 = x_183; +x_22 = x_184; +goto block_29; +} +} +} +else +{ +lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; +lean_dec(x_147); +lean_dec(x_142); +lean_dec(x_31); +lean_dec(x_32); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_185 = lean_ctor_get(x_162, 0); +lean_inc(x_185); +x_186 = lean_ctor_get(x_162, 1); +lean_inc(x_186); +if (lean_is_exclusive(x_162)) { + lean_ctor_release(x_162, 0); + lean_ctor_release(x_162, 1); + x_187 = x_162; +} else { + lean_dec_ref(x_162); + x_187 = lean_box(0); +} +if (lean_is_scalar(x_187)) { + x_188 = lean_alloc_ctor(1, 2, 0); +} else { + x_188 = x_187; +} +lean_ctor_set(x_188, 0, x_185); +lean_ctor_set(x_188, 1, x_186); +return x_188; +} +} +else +{ +lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; +lean_dec(x_144); +lean_dec(x_142); +lean_dec(x_31); +lean_dec(x_32); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_189 = lean_ctor_get(x_146, 0); +lean_inc(x_189); +x_190 = lean_ctor_get(x_146, 1); +lean_inc(x_190); +if (lean_is_exclusive(x_146)) { + lean_ctor_release(x_146, 0); + lean_ctor_release(x_146, 1); + x_191 = x_146; +} else { + lean_dec_ref(x_146); + x_191 = lean_box(0); } -if (lean_is_scalar(x_135)) { - x_136 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_191)) { + x_192 = lean_alloc_ctor(1, 2, 0); } else { - x_136 = x_135; + x_192 = x_191; } -lean_ctor_set(x_136, 0, x_133); -lean_ctor_set(x_136, 1, x_134); -return x_136; +lean_ctor_set(x_192, 0, x_189); +lean_ctor_set(x_192, 1, x_190); +return x_192; } } else { -lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; -lean_dec(x_95); -lean_dec(x_30); +lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; +lean_dec(x_142); lean_dec(x_31); +lean_dec(x_32); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -42426,39 +43010,40 @@ lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_137 = lean_ctor_get(x_96, 0); -lean_inc(x_137); -x_138 = lean_ctor_get(x_96, 1); -lean_inc(x_138); -if (lean_is_exclusive(x_96)) { - lean_ctor_release(x_96, 0); - lean_ctor_release(x_96, 1); - x_139 = x_96; +x_193 = lean_ctor_get(x_143, 0); +lean_inc(x_193); +x_194 = lean_ctor_get(x_143, 1); +lean_inc(x_194); +if (lean_is_exclusive(x_143)) { + lean_ctor_release(x_143, 0); + lean_ctor_release(x_143, 1); + x_195 = x_143; } else { - lean_dec_ref(x_96); - x_139 = lean_box(0); + lean_dec_ref(x_143); + x_195 = lean_box(0); } -if (lean_is_scalar(x_139)) { - x_140 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_195)) { + x_196 = lean_alloc_ctor(1, 2, 0); } else { - x_140 = x_139; + x_196 = x_195; } -lean_ctor_set(x_140, 0, x_137); -lean_ctor_set(x_140, 1, x_138); -return x_140; +lean_ctor_set(x_196, 0, x_193); +lean_ctor_set(x_196, 1, x_194); +return x_196; } } } else { -uint8_t x_141; -lean_dec(x_30); -lean_dec(x_41); +uint8_t x_197; lean_dec(x_31); +lean_dec(x_42); +lean_dec(x_32); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -42466,63 +43051,64 @@ lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_141 = !lean_is_exclusive(x_44); -if (x_141 == 0) +x_197 = !lean_is_exclusive(x_45); +if (x_197 == 0) { -return x_44; +return x_45; } else { -lean_object* x_142; lean_object* x_143; lean_object* x_144; -x_142 = lean_ctor_get(x_44, 0); -x_143 = lean_ctor_get(x_44, 1); -lean_inc(x_143); -lean_inc(x_142); -lean_dec(x_44); -x_144 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_144, 0, x_142); -lean_ctor_set(x_144, 1, x_143); -return x_144; +lean_object* x_198; lean_object* x_199; lean_object* x_200; +x_198 = lean_ctor_get(x_45, 0); +x_199 = lean_ctor_get(x_45, 1); +lean_inc(x_199); +lean_inc(x_198); +lean_dec(x_45); +x_200 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_200, 0, x_198); +lean_ctor_set(x_200, 1, x_199); +return x_200; } } } else { -lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; -lean_dec(x_30); -x_145 = lean_array_fget(x_32, x_33); -x_146 = lean_unsigned_to_nat(1u); -x_147 = lean_nat_add(x_33, x_146); -lean_dec(x_33); -x_148 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_148, 0, x_32); -lean_ctor_set(x_148, 1, x_147); -lean_ctor_set(x_148, 2, x_34); -x_149 = l___private_Lean_Elab_Tactic_BuiltinTactic_0__Lean_Elab_Tactic_getCaseGoals(x_19, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_149) == 0) -{ -lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; -x_150 = lean_ctor_get(x_149, 0); -lean_inc(x_150); -x_151 = lean_ctor_get(x_149, 1); -lean_inc(x_151); -lean_dec(x_149); -x_152 = lean_ctor_get(x_150, 0); -lean_inc(x_152); -x_153 = lean_ctor_get(x_150, 1); -lean_inc(x_153); -if (lean_is_exclusive(x_150)) { - lean_ctor_release(x_150, 0); - lean_ctor_release(x_150, 1); - x_154 = x_150; +lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; +lean_dec(x_31); +x_201 = lean_array_fget(x_33, x_34); +x_202 = lean_unsigned_to_nat(1u); +x_203 = lean_nat_add(x_34, x_202); +lean_dec(x_34); +x_204 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_204, 0, x_33); +lean_ctor_set(x_204, 1, x_203); +lean_ctor_set(x_204, 2, x_35); +x_205 = l___private_Lean_Elab_Tactic_BuiltinTactic_0__Lean_Elab_Tactic_getCaseGoals(x_20, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +if (lean_obj_tag(x_205) == 0) +{ +lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; +x_206 = lean_ctor_get(x_205, 0); +lean_inc(x_206); +x_207 = lean_ctor_get(x_205, 1); +lean_inc(x_207); +lean_dec(x_205); +x_208 = lean_ctor_get(x_206, 0); +lean_inc(x_208); +x_209 = lean_ctor_get(x_206, 1); +lean_inc(x_209); +if (lean_is_exclusive(x_206)) { + lean_ctor_release(x_206, 0); + lean_ctor_release(x_206, 1); + x_210 = x_206; } else { - lean_dec_ref(x_150); - x_154 = lean_box(0); + lean_dec_ref(x_206); + x_210 = lean_box(0); } +lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); @@ -42530,42 +43116,73 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); -x_155 = l_Lean_Elab_Tactic_renameInaccessibles(x_152, x_145, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_151); -if (lean_obj_tag(x_155) == 0) +x_211 = l_Lean_Elab_Tactic_renameInaccessibles(x_208, x_201, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_207); +if (lean_obj_tag(x_211) == 0) { -lean_object* x_156; lean_object* x_157; lean_object* x_158; -x_156 = lean_ctor_get(x_155, 0); -lean_inc(x_156); -x_157 = lean_ctor_get(x_155, 1); -lean_inc(x_157); -lean_dec(x_155); -lean_inc(x_156); -x_158 = l_Lean_MVarId_getTag(x_156, x_12, x_13, x_14, x_15, x_157); -if (lean_obj_tag(x_158) == 0) +lean_object* x_212; lean_object* x_213; lean_object* x_214; +x_212 = lean_ctor_get(x_211, 0); +lean_inc(x_212); +x_213 = lean_ctor_get(x_211, 1); +lean_inc(x_213); +lean_dec(x_211); +lean_inc(x_212); +x_214 = l_Lean_MVarId_getTag(x_212, x_13, x_14, x_15, x_16, x_213); +if (lean_obj_tag(x_214) == 0) { -lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; -x_159 = lean_ctor_get(x_158, 0); -lean_inc(x_159); -x_160 = lean_ctor_get(x_158, 1); -lean_inc(x_160); -lean_dec(x_158); -lean_inc(x_3); -if (lean_is_scalar(x_154)) { - x_161 = lean_alloc_ctor(1, 2, 0); +lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; +x_215 = lean_ctor_get(x_214, 0); +lean_inc(x_215); +x_216 = lean_ctor_get(x_214, 1); +lean_inc(x_216); +lean_dec(x_214); +lean_inc(x_4); +if (lean_is_scalar(x_210)) { + x_217 = lean_alloc_ctor(1, 2, 0); } else { - x_161 = x_154; - lean_ctor_set_tag(x_161, 1); + x_217 = x_210; + lean_ctor_set_tag(x_217, 1); } -lean_ctor_set(x_161, 0, x_156); -lean_ctor_set(x_161, 1, x_3); -x_162 = l_Lean_Elab_Tactic_setGoals(x_161, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_160); -x_163 = lean_ctor_get(x_162, 1); -lean_inc(x_163); -lean_dec(x_162); +lean_ctor_set(x_217, 0, x_212); +lean_ctor_set(x_217, 1, x_4); +x_218 = l_Lean_Elab_Tactic_setGoals(x_217, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_216); +x_219 = lean_ctor_get(x_218, 1); +lean_inc(x_219); +if (lean_is_exclusive(x_218)) { + lean_ctor_release(x_218, 0); + lean_ctor_release(x_218, 1); + x_220 = x_218; +} else { + lean_dec_ref(x_218); + x_220 = lean_box(0); +} +x_221 = lean_box(0); lean_inc(x_2); -x_164 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalTactic), 10, 1); -lean_closure_set(x_164, 0, x_2); +if (lean_is_scalar(x_220)) { + x_222 = lean_alloc_ctor(1, 2, 0); +} else { + x_222 = x_220; + lean_ctor_set_tag(x_222, 1); +} +lean_ctor_set(x_222, 0, x_2); +lean_ctor_set(x_222, 1, x_221); +lean_inc(x_1); +x_223 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_223, 0, x_1); +lean_ctor_set(x_223, 1, x_222); +x_224 = lean_array_mk(x_223); +x_225 = lean_box(2); +x_226 = l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1___lambda__1___closed__2; +x_227 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_227, 0, x_225); +lean_ctor_set(x_227, 1, x_226); +lean_ctor_set(x_227, 2, x_224); +lean_inc(x_3); +x_228 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalTactic), 10, 1); +lean_closure_set(x_228, 0, x_3); +x_229 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); +lean_closure_set(x_229, 0, x_227); +lean_closure_set(x_229, 1, x_228); +lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); @@ -42573,95 +43190,95 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); +lean_inc(x_3); lean_inc(x_2); -lean_inc(x_1); -x_165 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalCase___spec__5(x_1, x_2, x_164, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_163); -if (lean_obj_tag(x_165) == 0) +x_230 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalCase___spec__5(x_2, x_3, x_229, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_219); +if (lean_obj_tag(x_230) == 0) { -lean_object* x_166; lean_object* x_167; lean_object* x_168; -x_166 = lean_ctor_get(x_165, 1); -lean_inc(x_166); -lean_dec(x_165); -x_167 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_166); -x_168 = lean_ctor_get(x_167, 0); -lean_inc(x_168); -if (lean_obj_tag(x_168) == 0) +lean_object* x_231; lean_object* x_232; lean_object* x_233; +x_231 = lean_ctor_get(x_230, 1); +lean_inc(x_231); +lean_dec(x_230); +x_232 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_231); +x_233 = lean_ctor_get(x_232, 0); +lean_inc(x_233); +if (lean_obj_tag(x_233) == 0) { -lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; -lean_dec(x_159); -x_169 = lean_ctor_get(x_167, 1); -lean_inc(x_169); -lean_dec(x_167); -x_170 = lean_box(0); -x_171 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_168, x_153, x_148, x_31, x_170, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_169); -x_172 = lean_ctor_get(x_171, 0); -lean_inc(x_172); -x_173 = lean_ctor_get(x_171, 1); -lean_inc(x_173); -lean_dec(x_171); -x_20 = x_172; -x_21 = x_173; -goto block_28; +lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; +lean_dec(x_215); +x_234 = lean_ctor_get(x_232, 1); +lean_inc(x_234); +lean_dec(x_232); +x_235 = lean_box(0); +x_236 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_233, x_209, x_204, x_32, x_235, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_234); +x_237 = lean_ctor_get(x_236, 0); +lean_inc(x_237); +x_238 = lean_ctor_get(x_236, 1); +lean_inc(x_238); +lean_dec(x_236); +x_21 = x_237; +x_22 = x_238; +goto block_29; } else { -lean_object* x_174; -x_174 = lean_ctor_get(x_168, 1); -lean_inc(x_174); -if (lean_obj_tag(x_174) == 0) +lean_object* x_239; +x_239 = lean_ctor_get(x_233, 1); +lean_inc(x_239); +if (lean_obj_tag(x_239) == 0) { -lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; -x_175 = lean_ctor_get(x_167, 1); -lean_inc(x_175); -lean_dec(x_167); -x_176 = lean_ctor_get(x_168, 0); -lean_inc(x_176); -x_177 = l_Lean_MVarId_setTag(x_176, x_159, x_12, x_13, x_14, x_15, x_175); -x_178 = lean_ctor_get(x_177, 0); -lean_inc(x_178); -x_179 = lean_ctor_get(x_177, 1); -lean_inc(x_179); -lean_dec(x_177); -x_180 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_168, x_153, x_148, x_31, x_178, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_179); -lean_dec(x_178); -x_181 = lean_ctor_get(x_180, 0); -lean_inc(x_181); -x_182 = lean_ctor_get(x_180, 1); -lean_inc(x_182); -lean_dec(x_180); -x_20 = x_181; -x_21 = x_182; -goto block_28; +lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; +x_240 = lean_ctor_get(x_232, 1); +lean_inc(x_240); +lean_dec(x_232); +x_241 = lean_ctor_get(x_233, 0); +lean_inc(x_241); +x_242 = l_Lean_MVarId_setTag(x_241, x_215, x_13, x_14, x_15, x_16, x_240); +x_243 = lean_ctor_get(x_242, 0); +lean_inc(x_243); +x_244 = lean_ctor_get(x_242, 1); +lean_inc(x_244); +lean_dec(x_242); +x_245 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_233, x_209, x_204, x_32, x_243, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_244); +lean_dec(x_243); +x_246 = lean_ctor_get(x_245, 0); +lean_inc(x_246); +x_247 = lean_ctor_get(x_245, 1); +lean_inc(x_247); +lean_dec(x_245); +x_21 = x_246; +x_22 = x_247; +goto block_29; } else { -lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; -lean_dec(x_174); -lean_dec(x_159); -x_183 = lean_ctor_get(x_167, 1); -lean_inc(x_183); -lean_dec(x_167); -x_184 = lean_box(0); -x_185 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_168, x_153, x_148, x_31, x_184, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_183); -x_186 = lean_ctor_get(x_185, 0); -lean_inc(x_186); -x_187 = lean_ctor_get(x_185, 1); -lean_inc(x_187); -lean_dec(x_185); -x_20 = x_186; -x_21 = x_187; -goto block_28; +lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; +lean_dec(x_239); +lean_dec(x_215); +x_248 = lean_ctor_get(x_232, 1); +lean_inc(x_248); +lean_dec(x_232); +x_249 = lean_box(0); +x_250 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_233, x_209, x_204, x_32, x_249, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_248); +x_251 = lean_ctor_get(x_250, 0); +lean_inc(x_251); +x_252 = lean_ctor_get(x_250, 1); +lean_inc(x_252); +lean_dec(x_250); +x_21 = x_251; +x_22 = x_252; +goto block_29; } } } else { -lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; -lean_dec(x_159); -lean_dec(x_153); -lean_dec(x_148); -lean_dec(x_31); +lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; +lean_dec(x_215); +lean_dec(x_209); +lean_dec(x_204); +lean_dec(x_32); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -42669,40 +43286,41 @@ lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_188 = lean_ctor_get(x_165, 0); -lean_inc(x_188); -x_189 = lean_ctor_get(x_165, 1); -lean_inc(x_189); -if (lean_is_exclusive(x_165)) { - lean_ctor_release(x_165, 0); - lean_ctor_release(x_165, 1); - x_190 = x_165; +x_253 = lean_ctor_get(x_230, 0); +lean_inc(x_253); +x_254 = lean_ctor_get(x_230, 1); +lean_inc(x_254); +if (lean_is_exclusive(x_230)) { + lean_ctor_release(x_230, 0); + lean_ctor_release(x_230, 1); + x_255 = x_230; } else { - lean_dec_ref(x_165); - x_190 = lean_box(0); + lean_dec_ref(x_230); + x_255 = lean_box(0); } -if (lean_is_scalar(x_190)) { - x_191 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_255)) { + x_256 = lean_alloc_ctor(1, 2, 0); } else { - x_191 = x_190; + x_256 = x_255; } -lean_ctor_set(x_191, 0, x_188); -lean_ctor_set(x_191, 1, x_189); -return x_191; +lean_ctor_set(x_256, 0, x_253); +lean_ctor_set(x_256, 1, x_254); +return x_256; } } else { -lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; -lean_dec(x_156); -lean_dec(x_154); -lean_dec(x_153); -lean_dec(x_148); -lean_dec(x_31); +lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; +lean_dec(x_212); +lean_dec(x_210); +lean_dec(x_209); +lean_dec(x_204); +lean_dec(x_32); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -42710,39 +43328,40 @@ lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_192 = lean_ctor_get(x_158, 0); -lean_inc(x_192); -x_193 = lean_ctor_get(x_158, 1); -lean_inc(x_193); -if (lean_is_exclusive(x_158)) { - lean_ctor_release(x_158, 0); - lean_ctor_release(x_158, 1); - x_194 = x_158; +x_257 = lean_ctor_get(x_214, 0); +lean_inc(x_257); +x_258 = lean_ctor_get(x_214, 1); +lean_inc(x_258); +if (lean_is_exclusive(x_214)) { + lean_ctor_release(x_214, 0); + lean_ctor_release(x_214, 1); + x_259 = x_214; } else { - lean_dec_ref(x_158); - x_194 = lean_box(0); + lean_dec_ref(x_214); + x_259 = lean_box(0); } -if (lean_is_scalar(x_194)) { - x_195 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_259)) { + x_260 = lean_alloc_ctor(1, 2, 0); } else { - x_195 = x_194; + x_260 = x_259; } -lean_ctor_set(x_195, 0, x_192); -lean_ctor_set(x_195, 1, x_193); -return x_195; +lean_ctor_set(x_260, 0, x_257); +lean_ctor_set(x_260, 1, x_258); +return x_260; } } else { -lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; -lean_dec(x_154); -lean_dec(x_153); -lean_dec(x_148); -lean_dec(x_31); +lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; +lean_dec(x_210); +lean_dec(x_209); +lean_dec(x_204); +lean_dec(x_32); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -42750,38 +43369,39 @@ lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_196 = lean_ctor_get(x_155, 0); -lean_inc(x_196); -x_197 = lean_ctor_get(x_155, 1); -lean_inc(x_197); -if (lean_is_exclusive(x_155)) { - lean_ctor_release(x_155, 0); - lean_ctor_release(x_155, 1); - x_198 = x_155; +x_261 = lean_ctor_get(x_211, 0); +lean_inc(x_261); +x_262 = lean_ctor_get(x_211, 1); +lean_inc(x_262); +if (lean_is_exclusive(x_211)) { + lean_ctor_release(x_211, 0); + lean_ctor_release(x_211, 1); + x_263 = x_211; } else { - lean_dec_ref(x_155); - x_198 = lean_box(0); + lean_dec_ref(x_211); + x_263 = lean_box(0); } -if (lean_is_scalar(x_198)) { - x_199 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_263)) { + x_264 = lean_alloc_ctor(1, 2, 0); } else { - x_199 = x_198; + x_264 = x_263; } -lean_ctor_set(x_199, 0, x_196); -lean_ctor_set(x_199, 1, x_197); -return x_199; +lean_ctor_set(x_264, 0, x_261); +lean_ctor_set(x_264, 1, x_262); +return x_264; } } else { -lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; -lean_dec(x_148); -lean_dec(x_145); -lean_dec(x_31); +lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; +lean_dec(x_204); +lean_dec(x_201); +lean_dec(x_32); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -42789,110 +43409,111 @@ lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_200 = lean_ctor_get(x_149, 0); -lean_inc(x_200); -x_201 = lean_ctor_get(x_149, 1); -lean_inc(x_201); -if (lean_is_exclusive(x_149)) { - lean_ctor_release(x_149, 0); - lean_ctor_release(x_149, 1); - x_202 = x_149; +x_265 = lean_ctor_get(x_205, 0); +lean_inc(x_265); +x_266 = lean_ctor_get(x_205, 1); +lean_inc(x_266); +if (lean_is_exclusive(x_205)) { + lean_ctor_release(x_205, 0); + lean_ctor_release(x_205, 1); + x_267 = x_205; } else { - lean_dec_ref(x_149); - x_202 = lean_box(0); + lean_dec_ref(x_205); + x_267 = lean_box(0); } -if (lean_is_scalar(x_202)) { - x_203 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_267)) { + x_268 = lean_alloc_ctor(1, 2, 0); } else { - x_203 = x_202; + x_268 = x_267; } -lean_ctor_set(x_203, 0, x_200); -lean_ctor_set(x_203, 1, x_201); -return x_203; +lean_ctor_set(x_268, 0, x_265); +lean_ctor_set(x_268, 1, x_266); +return x_268; } } } } else { -lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; uint8_t x_209; -x_204 = lean_ctor_get(x_7, 0); -x_205 = lean_ctor_get(x_7, 1); -lean_inc(x_205); -lean_inc(x_204); -lean_dec(x_7); -x_206 = lean_ctor_get(x_204, 0); -lean_inc(x_206); -x_207 = lean_ctor_get(x_204, 1); -lean_inc(x_207); -x_208 = lean_ctor_get(x_204, 2); -lean_inc(x_208); -x_209 = lean_nat_dec_lt(x_207, x_208); -if (x_209 == 0) +lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; uint8_t x_274; +x_269 = lean_ctor_get(x_8, 0); +x_270 = lean_ctor_get(x_8, 1); +lean_inc(x_270); +lean_inc(x_269); +lean_dec(x_8); +x_271 = lean_ctor_get(x_269, 0); +lean_inc(x_271); +x_272 = lean_ctor_get(x_269, 1); +lean_inc(x_272); +x_273 = lean_ctor_get(x_269, 2); +lean_inc(x_273); +x_274 = lean_nat_dec_lt(x_272, x_273); +if (x_274 == 0) { -lean_object* x_210; lean_object* x_211; -lean_dec(x_208); -lean_dec(x_207); -lean_dec(x_206); -lean_dec(x_19); -x_210 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_210, 0, x_204); -lean_ctor_set(x_210, 1, x_205); -x_211 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_211, 0, x_210); -x_20 = x_211; -x_21 = x_16; -goto block_28; +lean_object* x_275; lean_object* x_276; +lean_dec(x_273); +lean_dec(x_272); +lean_dec(x_271); +lean_dec(x_20); +x_275 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_275, 0, x_269); +lean_ctor_set(x_275, 1, x_270); +x_276 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_276, 0, x_275); +x_21 = x_276; +x_22 = x_17; +goto block_29; } else { -lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; -if (lean_is_exclusive(x_204)) { - lean_ctor_release(x_204, 0); - lean_ctor_release(x_204, 1); - lean_ctor_release(x_204, 2); - x_212 = x_204; +lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; +if (lean_is_exclusive(x_269)) { + lean_ctor_release(x_269, 0); + lean_ctor_release(x_269, 1); + lean_ctor_release(x_269, 2); + x_277 = x_269; } else { - lean_dec_ref(x_204); - x_212 = lean_box(0); + lean_dec_ref(x_269); + x_277 = lean_box(0); } -x_213 = lean_array_fget(x_206, x_207); -x_214 = lean_unsigned_to_nat(1u); -x_215 = lean_nat_add(x_207, x_214); -lean_dec(x_207); -if (lean_is_scalar(x_212)) { - x_216 = lean_alloc_ctor(0, 3, 0); +x_278 = lean_array_fget(x_271, x_272); +x_279 = lean_unsigned_to_nat(1u); +x_280 = lean_nat_add(x_272, x_279); +lean_dec(x_272); +if (lean_is_scalar(x_277)) { + x_281 = lean_alloc_ctor(0, 3, 0); } else { - x_216 = x_212; + x_281 = x_277; } -lean_ctor_set(x_216, 0, x_206); -lean_ctor_set(x_216, 1, x_215); -lean_ctor_set(x_216, 2, x_208); -x_217 = l___private_Lean_Elab_Tactic_BuiltinTactic_0__Lean_Elab_Tactic_getCaseGoals(x_19, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_217) == 0) -{ -lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; -x_218 = lean_ctor_get(x_217, 0); -lean_inc(x_218); -x_219 = lean_ctor_get(x_217, 1); -lean_inc(x_219); -lean_dec(x_217); -x_220 = lean_ctor_get(x_218, 0); -lean_inc(x_220); -x_221 = lean_ctor_get(x_218, 1); -lean_inc(x_221); -if (lean_is_exclusive(x_218)) { - lean_ctor_release(x_218, 0); - lean_ctor_release(x_218, 1); - x_222 = x_218; +lean_ctor_set(x_281, 0, x_271); +lean_ctor_set(x_281, 1, x_280); +lean_ctor_set(x_281, 2, x_273); +x_282 = l___private_Lean_Elab_Tactic_BuiltinTactic_0__Lean_Elab_Tactic_getCaseGoals(x_20, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +if (lean_obj_tag(x_282) == 0) +{ +lean_object* x_283; lean_object* x_284; lean_object* x_285; lean_object* x_286; lean_object* x_287; lean_object* x_288; +x_283 = lean_ctor_get(x_282, 0); +lean_inc(x_283); +x_284 = lean_ctor_get(x_282, 1); +lean_inc(x_284); +lean_dec(x_282); +x_285 = lean_ctor_get(x_283, 0); +lean_inc(x_285); +x_286 = lean_ctor_get(x_283, 1); +lean_inc(x_286); +if (lean_is_exclusive(x_283)) { + lean_ctor_release(x_283, 0); + lean_ctor_release(x_283, 1); + x_287 = x_283; } else { - lean_dec_ref(x_218); - x_222 = lean_box(0); + lean_dec_ref(x_283); + x_287 = lean_box(0); } +lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); @@ -42900,42 +43521,73 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); -x_223 = l_Lean_Elab_Tactic_renameInaccessibles(x_220, x_213, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_219); -if (lean_obj_tag(x_223) == 0) -{ -lean_object* x_224; lean_object* x_225; lean_object* x_226; -x_224 = lean_ctor_get(x_223, 0); -lean_inc(x_224); -x_225 = lean_ctor_get(x_223, 1); -lean_inc(x_225); -lean_dec(x_223); -lean_inc(x_224); -x_226 = l_Lean_MVarId_getTag(x_224, x_12, x_13, x_14, x_15, x_225); -if (lean_obj_tag(x_226) == 0) +x_288 = l_Lean_Elab_Tactic_renameInaccessibles(x_285, x_278, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_284); +if (lean_obj_tag(x_288) == 0) { -lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; -x_227 = lean_ctor_get(x_226, 0); -lean_inc(x_227); -x_228 = lean_ctor_get(x_226, 1); -lean_inc(x_228); -lean_dec(x_226); -lean_inc(x_3); -if (lean_is_scalar(x_222)) { - x_229 = lean_alloc_ctor(1, 2, 0); +lean_object* x_289; lean_object* x_290; lean_object* x_291; +x_289 = lean_ctor_get(x_288, 0); +lean_inc(x_289); +x_290 = lean_ctor_get(x_288, 1); +lean_inc(x_290); +lean_dec(x_288); +lean_inc(x_289); +x_291 = l_Lean_MVarId_getTag(x_289, x_13, x_14, x_15, x_16, x_290); +if (lean_obj_tag(x_291) == 0) +{ +lean_object* x_292; lean_object* x_293; lean_object* x_294; lean_object* x_295; lean_object* x_296; lean_object* x_297; lean_object* x_298; lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; lean_object* x_307; +x_292 = lean_ctor_get(x_291, 0); +lean_inc(x_292); +x_293 = lean_ctor_get(x_291, 1); +lean_inc(x_293); +lean_dec(x_291); +lean_inc(x_4); +if (lean_is_scalar(x_287)) { + x_294 = lean_alloc_ctor(1, 2, 0); +} else { + x_294 = x_287; + lean_ctor_set_tag(x_294, 1); +} +lean_ctor_set(x_294, 0, x_289); +lean_ctor_set(x_294, 1, x_4); +x_295 = l_Lean_Elab_Tactic_setGoals(x_294, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_293); +x_296 = lean_ctor_get(x_295, 1); +lean_inc(x_296); +if (lean_is_exclusive(x_295)) { + lean_ctor_release(x_295, 0); + lean_ctor_release(x_295, 1); + x_297 = x_295; +} else { + lean_dec_ref(x_295); + x_297 = lean_box(0); +} +x_298 = lean_box(0); +lean_inc(x_2); +if (lean_is_scalar(x_297)) { + x_299 = lean_alloc_ctor(1, 2, 0); } else { - x_229 = x_222; - lean_ctor_set_tag(x_229, 1); + x_299 = x_297; + lean_ctor_set_tag(x_299, 1); } -lean_ctor_set(x_229, 0, x_224); -lean_ctor_set(x_229, 1, x_3); -x_230 = l_Lean_Elab_Tactic_setGoals(x_229, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_228); -x_231 = lean_ctor_get(x_230, 1); -lean_inc(x_231); -lean_dec(x_230); -lean_inc(x_2); -x_232 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalTactic), 10, 1); -lean_closure_set(x_232, 0, x_2); +lean_ctor_set(x_299, 0, x_2); +lean_ctor_set(x_299, 1, x_298); +lean_inc(x_1); +x_300 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_300, 0, x_1); +lean_ctor_set(x_300, 1, x_299); +x_301 = lean_array_mk(x_300); +x_302 = lean_box(2); +x_303 = l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1___lambda__1___closed__2; +x_304 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_304, 0, x_302); +lean_ctor_set(x_304, 1, x_303); +lean_ctor_set(x_304, 2, x_301); +lean_inc(x_3); +x_305 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalTactic), 10, 1); +lean_closure_set(x_305, 0, x_3); +x_306 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); +lean_closure_set(x_306, 0, x_304); +lean_closure_set(x_306, 1, x_305); +lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); @@ -42943,95 +43595,95 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); +lean_inc(x_3); lean_inc(x_2); -lean_inc(x_1); -x_233 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalCase___spec__5(x_1, x_2, x_232, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_231); -if (lean_obj_tag(x_233) == 0) +x_307 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalCase___spec__5(x_2, x_3, x_306, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_296); +if (lean_obj_tag(x_307) == 0) { -lean_object* x_234; lean_object* x_235; lean_object* x_236; -x_234 = lean_ctor_get(x_233, 1); -lean_inc(x_234); -lean_dec(x_233); -x_235 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_234); -x_236 = lean_ctor_get(x_235, 0); -lean_inc(x_236); -if (lean_obj_tag(x_236) == 0) +lean_object* x_308; lean_object* x_309; lean_object* x_310; +x_308 = lean_ctor_get(x_307, 1); +lean_inc(x_308); +lean_dec(x_307); +x_309 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_308); +x_310 = lean_ctor_get(x_309, 0); +lean_inc(x_310); +if (lean_obj_tag(x_310) == 0) { -lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; -lean_dec(x_227); -x_237 = lean_ctor_get(x_235, 1); -lean_inc(x_237); -lean_dec(x_235); -x_238 = lean_box(0); -x_239 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_236, x_221, x_216, x_205, x_238, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_237); -x_240 = lean_ctor_get(x_239, 0); -lean_inc(x_240); -x_241 = lean_ctor_get(x_239, 1); -lean_inc(x_241); -lean_dec(x_239); -x_20 = x_240; -x_21 = x_241; -goto block_28; +lean_object* x_311; lean_object* x_312; lean_object* x_313; lean_object* x_314; lean_object* x_315; +lean_dec(x_292); +x_311 = lean_ctor_get(x_309, 1); +lean_inc(x_311); +lean_dec(x_309); +x_312 = lean_box(0); +x_313 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_310, x_286, x_281, x_270, x_312, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_311); +x_314 = lean_ctor_get(x_313, 0); +lean_inc(x_314); +x_315 = lean_ctor_get(x_313, 1); +lean_inc(x_315); +lean_dec(x_313); +x_21 = x_314; +x_22 = x_315; +goto block_29; } else { -lean_object* x_242; -x_242 = lean_ctor_get(x_236, 1); -lean_inc(x_242); -if (lean_obj_tag(x_242) == 0) +lean_object* x_316; +x_316 = lean_ctor_get(x_310, 1); +lean_inc(x_316); +if (lean_obj_tag(x_316) == 0) { -lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; -x_243 = lean_ctor_get(x_235, 1); -lean_inc(x_243); -lean_dec(x_235); -x_244 = lean_ctor_get(x_236, 0); -lean_inc(x_244); -x_245 = l_Lean_MVarId_setTag(x_244, x_227, x_12, x_13, x_14, x_15, x_243); -x_246 = lean_ctor_get(x_245, 0); -lean_inc(x_246); -x_247 = lean_ctor_get(x_245, 1); -lean_inc(x_247); -lean_dec(x_245); -x_248 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_236, x_221, x_216, x_205, x_246, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_247); -lean_dec(x_246); -x_249 = lean_ctor_get(x_248, 0); -lean_inc(x_249); -x_250 = lean_ctor_get(x_248, 1); -lean_inc(x_250); -lean_dec(x_248); -x_20 = x_249; -x_21 = x_250; -goto block_28; +lean_object* x_317; lean_object* x_318; lean_object* x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; lean_object* x_324; +x_317 = lean_ctor_get(x_309, 1); +lean_inc(x_317); +lean_dec(x_309); +x_318 = lean_ctor_get(x_310, 0); +lean_inc(x_318); +x_319 = l_Lean_MVarId_setTag(x_318, x_292, x_13, x_14, x_15, x_16, x_317); +x_320 = lean_ctor_get(x_319, 0); +lean_inc(x_320); +x_321 = lean_ctor_get(x_319, 1); +lean_inc(x_321); +lean_dec(x_319); +x_322 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_310, x_286, x_281, x_270, x_320, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_321); +lean_dec(x_320); +x_323 = lean_ctor_get(x_322, 0); +lean_inc(x_323); +x_324 = lean_ctor_get(x_322, 1); +lean_inc(x_324); +lean_dec(x_322); +x_21 = x_323; +x_22 = x_324; +goto block_29; } else { -lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; -lean_dec(x_242); -lean_dec(x_227); -x_251 = lean_ctor_get(x_235, 1); -lean_inc(x_251); -lean_dec(x_235); -x_252 = lean_box(0); -x_253 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_236, x_221, x_216, x_205, x_252, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_251); -x_254 = lean_ctor_get(x_253, 0); -lean_inc(x_254); -x_255 = lean_ctor_get(x_253, 1); -lean_inc(x_255); -lean_dec(x_253); -x_20 = x_254; -x_21 = x_255; -goto block_28; +lean_object* x_325; lean_object* x_326; lean_object* x_327; lean_object* x_328; lean_object* x_329; +lean_dec(x_316); +lean_dec(x_292); +x_325 = lean_ctor_get(x_309, 1); +lean_inc(x_325); +lean_dec(x_309); +x_326 = lean_box(0); +x_327 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_310, x_286, x_281, x_270, x_326, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_325); +x_328 = lean_ctor_get(x_327, 0); +lean_inc(x_328); +x_329 = lean_ctor_get(x_327, 1); +lean_inc(x_329); +lean_dec(x_327); +x_21 = x_328; +x_22 = x_329; +goto block_29; } } } else { -lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; -lean_dec(x_227); -lean_dec(x_221); -lean_dec(x_216); -lean_dec(x_205); +lean_object* x_330; lean_object* x_331; lean_object* x_332; lean_object* x_333; +lean_dec(x_292); +lean_dec(x_286); +lean_dec(x_281); +lean_dec(x_270); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -43039,40 +43691,41 @@ lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_256 = lean_ctor_get(x_233, 0); -lean_inc(x_256); -x_257 = lean_ctor_get(x_233, 1); -lean_inc(x_257); -if (lean_is_exclusive(x_233)) { - lean_ctor_release(x_233, 0); - lean_ctor_release(x_233, 1); - x_258 = x_233; +x_330 = lean_ctor_get(x_307, 0); +lean_inc(x_330); +x_331 = lean_ctor_get(x_307, 1); +lean_inc(x_331); +if (lean_is_exclusive(x_307)) { + lean_ctor_release(x_307, 0); + lean_ctor_release(x_307, 1); + x_332 = x_307; } else { - lean_dec_ref(x_233); - x_258 = lean_box(0); + lean_dec_ref(x_307); + x_332 = lean_box(0); } -if (lean_is_scalar(x_258)) { - x_259 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_332)) { + x_333 = lean_alloc_ctor(1, 2, 0); } else { - x_259 = x_258; + x_333 = x_332; } -lean_ctor_set(x_259, 0, x_256); -lean_ctor_set(x_259, 1, x_257); -return x_259; +lean_ctor_set(x_333, 0, x_330); +lean_ctor_set(x_333, 1, x_331); +return x_333; } } else { -lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; -lean_dec(x_224); -lean_dec(x_222); -lean_dec(x_221); -lean_dec(x_216); -lean_dec(x_205); +lean_object* x_334; lean_object* x_335; lean_object* x_336; lean_object* x_337; +lean_dec(x_289); +lean_dec(x_287); +lean_dec(x_286); +lean_dec(x_281); +lean_dec(x_270); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -43080,39 +43733,40 @@ lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_260 = lean_ctor_get(x_226, 0); -lean_inc(x_260); -x_261 = lean_ctor_get(x_226, 1); -lean_inc(x_261); -if (lean_is_exclusive(x_226)) { - lean_ctor_release(x_226, 0); - lean_ctor_release(x_226, 1); - x_262 = x_226; +x_334 = lean_ctor_get(x_291, 0); +lean_inc(x_334); +x_335 = lean_ctor_get(x_291, 1); +lean_inc(x_335); +if (lean_is_exclusive(x_291)) { + lean_ctor_release(x_291, 0); + lean_ctor_release(x_291, 1); + x_336 = x_291; } else { - lean_dec_ref(x_226); - x_262 = lean_box(0); + lean_dec_ref(x_291); + x_336 = lean_box(0); } -if (lean_is_scalar(x_262)) { - x_263 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_336)) { + x_337 = lean_alloc_ctor(1, 2, 0); } else { - x_263 = x_262; + x_337 = x_336; } -lean_ctor_set(x_263, 0, x_260); -lean_ctor_set(x_263, 1, x_261); -return x_263; +lean_ctor_set(x_337, 0, x_334); +lean_ctor_set(x_337, 1, x_335); +return x_337; } } else { -lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; -lean_dec(x_222); -lean_dec(x_221); -lean_dec(x_216); -lean_dec(x_205); +lean_object* x_338; lean_object* x_339; lean_object* x_340; lean_object* x_341; +lean_dec(x_287); +lean_dec(x_286); +lean_dec(x_281); +lean_dec(x_270); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -43120,38 +43774,39 @@ lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_264 = lean_ctor_get(x_223, 0); -lean_inc(x_264); -x_265 = lean_ctor_get(x_223, 1); -lean_inc(x_265); -if (lean_is_exclusive(x_223)) { - lean_ctor_release(x_223, 0); - lean_ctor_release(x_223, 1); - x_266 = x_223; +x_338 = lean_ctor_get(x_288, 0); +lean_inc(x_338); +x_339 = lean_ctor_get(x_288, 1); +lean_inc(x_339); +if (lean_is_exclusive(x_288)) { + lean_ctor_release(x_288, 0); + lean_ctor_release(x_288, 1); + x_340 = x_288; } else { - lean_dec_ref(x_223); - x_266 = lean_box(0); + lean_dec_ref(x_288); + x_340 = lean_box(0); } -if (lean_is_scalar(x_266)) { - x_267 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_340)) { + x_341 = lean_alloc_ctor(1, 2, 0); } else { - x_267 = x_266; + x_341 = x_340; } -lean_ctor_set(x_267, 0, x_264); -lean_ctor_set(x_267, 1, x_265); -return x_267; +lean_ctor_set(x_341, 0, x_338); +lean_ctor_set(x_341, 1, x_339); +return x_341; } } else { -lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; -lean_dec(x_216); -lean_dec(x_213); -lean_dec(x_205); +lean_object* x_342; lean_object* x_343; lean_object* x_344; lean_object* x_345; +lean_dec(x_281); +lean_dec(x_278); +lean_dec(x_270); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -43159,38 +43814,39 @@ lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_268 = lean_ctor_get(x_217, 0); -lean_inc(x_268); -x_269 = lean_ctor_get(x_217, 1); -lean_inc(x_269); -if (lean_is_exclusive(x_217)) { - lean_ctor_release(x_217, 0); - lean_ctor_release(x_217, 1); - x_270 = x_217; +x_342 = lean_ctor_get(x_282, 0); +lean_inc(x_342); +x_343 = lean_ctor_get(x_282, 1); +lean_inc(x_343); +if (lean_is_exclusive(x_282)) { + lean_ctor_release(x_282, 0); + lean_ctor_release(x_282, 1); + x_344 = x_282; } else { - lean_dec_ref(x_217); - x_270 = lean_box(0); + lean_dec_ref(x_282); + x_344 = lean_box(0); } -if (lean_is_scalar(x_270)) { - x_271 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_344)) { + x_345 = lean_alloc_ctor(1, 2, 0); } else { - x_271 = x_270; + x_345 = x_344; } -lean_ctor_set(x_271, 0, x_268); -lean_ctor_set(x_271, 1, x_269); -return x_271; +lean_ctor_set(x_345, 0, x_342); +lean_ctor_set(x_345, 1, x_343); +return x_345; } } } -block_28: +block_29: { -if (lean_obj_tag(x_20) == 0) +if (lean_obj_tag(x_21) == 0) { -lean_object* x_22; lean_object* x_23; +lean_object* x_23; lean_object* x_24; +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -43198,29 +43854,29 @@ lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_22 = lean_ctor_get(x_20, 0); -lean_inc(x_22); -lean_dec(x_20); -x_23 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_23, 0, x_22); -lean_ctor_set(x_23, 1, x_21); -return x_23; +x_23 = lean_ctor_get(x_21, 0); +lean_inc(x_23); +lean_dec(x_21); +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_23); +lean_ctor_set(x_24, 1, x_22); +return x_24; } else { -lean_object* x_24; size_t x_25; size_t x_26; -x_24 = lean_ctor_get(x_20, 0); -lean_inc(x_24); -lean_dec(x_20); -x_25 = 1; -x_26 = lean_usize_add(x_6, x_25); -x_6 = x_26; -x_7 = x_24; -x_16 = x_21; +lean_object* x_25; size_t x_26; size_t x_27; +x_25 = lean_ctor_get(x_21, 0); +lean_inc(x_25); +lean_dec(x_21); +x_26 = 1; +x_27 = lean_usize_add(x_7, x_26); +x_7 = x_27; +x_8 = x_25; +x_17 = x_22; goto _start; } } @@ -43271,61 +43927,63 @@ return x_13; } else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; -x_14 = lean_unsigned_to_nat(1u); +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; lean_object* x_21; +x_14 = lean_unsigned_to_nat(0u); x_15 = l_Lean_Syntax_getArg(x_1, x_14); -x_16 = l_Lean_Syntax_getArgs(x_15); -lean_dec(x_15); -x_17 = lean_array_get_size(x_16); -x_18 = lean_unsigned_to_nat(0u); -x_19 = lean_nat_dec_lt(x_18, x_17); -if (x_19 == 0) -{ -lean_object* x_57; +x_16 = lean_unsigned_to_nat(1u); +x_17 = l_Lean_Syntax_getArg(x_1, x_16); +x_18 = l_Lean_Syntax_getArgs(x_17); lean_dec(x_17); -lean_dec(x_16); -x_57 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Tactic_evalOpen___spec__3___closed__12; -x_20 = x_57; -goto block_56; +x_19 = lean_array_get_size(x_18); +x_20 = lean_nat_dec_lt(x_14, x_19); +if (x_20 == 0) +{ +lean_object* x_58; +lean_dec(x_19); +lean_dec(x_18); +x_58 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Tactic_evalOpen___spec__3___closed__12; +x_21 = x_58; +goto block_57; } else { -uint8_t x_58; -x_58 = lean_nat_dec_le(x_17, x_17); -if (x_58 == 0) +uint8_t x_59; +x_59 = lean_nat_dec_le(x_19, x_19); +if (x_59 == 0) { -lean_object* x_59; -lean_dec(x_17); -lean_dec(x_16); -x_59 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Tactic_evalOpen___spec__3___closed__12; -x_20 = x_59; -goto block_56; +lean_object* x_60; +lean_dec(x_19); +lean_dec(x_18); +x_60 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Tactic_evalOpen___spec__3___closed__12; +x_21 = x_60; +goto block_57; } else { -size_t x_60; size_t x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; -x_60 = 0; -x_61 = lean_usize_of_nat(x_17); -lean_dec(x_17); -x_62 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Tactic_evalOpen___spec__3___closed__13; -x_63 = l_Array_foldlMUnsafe_fold___at_Lean_Syntax_SepArray_getElems___spec__1(x_16, x_60, x_61, x_62); -lean_dec(x_16); -x_64 = lean_ctor_get(x_63, 1); -lean_inc(x_64); -lean_dec(x_63); -x_20 = x_64; -goto block_56; +size_t x_61; size_t x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_61 = 0; +x_62 = lean_usize_of_nat(x_19); +lean_dec(x_19); +x_63 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Tactic_evalOpen___spec__3___closed__13; +x_64 = l_Array_foldlMUnsafe_fold___at_Lean_Syntax_SepArray_getElems___spec__1(x_18, x_61, x_62, x_63); +lean_dec(x_18); +x_65 = lean_ctor_get(x_64, 1); +lean_inc(x_65); +lean_dec(x_64); +x_21 = x_65; +goto block_57; } } -block_56: +block_57: { -lean_object* x_21; lean_object* x_22; -x_21 = l_Lean_Elab_Tactic_evalCase___closed__3; -x_22 = l_Array_sequenceMap___at_Lean_Elab_Tactic_evalCase___spec__1(x_20, x_21); -lean_dec(x_20); -if (lean_obj_tag(x_22) == 0) +lean_object* x_22; lean_object* x_23; +x_22 = l_Lean_Elab_Tactic_evalCase___closed__3; +x_23 = l_Array_sequenceMap___at_Lean_Elab_Tactic_evalCase___spec__1(x_21, x_22); +lean_dec(x_21); +if (lean_obj_tag(x_23) == 0) { -lean_object* x_23; +lean_object* x_24; +lean_dec(x_15); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -43335,35 +43993,36 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_23 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(x_10); -return x_23; +x_24 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(x_10); +return x_24; } else { -lean_object* x_24; size_t x_25; size_t x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; -x_24 = lean_ctor_get(x_22, 0); -lean_inc(x_24); -lean_dec(x_22); -x_25 = lean_array_size(x_24); -x_26 = 0; -lean_inc(x_24); -x_27 = l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalCase___spec__3(x_25, x_26, x_24); -x_28 = l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalCase___spec__4(x_25, x_26, x_24); -x_29 = lean_unsigned_to_nat(2u); -x_30 = l_Lean_Syntax_getArg(x_1, x_29); -x_31 = lean_unsigned_to_nat(3u); -x_32 = l_Lean_Syntax_getArg(x_1, x_31); -lean_dec(x_1); -x_33 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_addCheckpoints___spec__1___closed__4; -lean_inc(x_32); -x_34 = l_Lean_Syntax_isOfKind(x_32, x_33); -if (x_34 == 0) +lean_object* x_25; size_t x_26; size_t x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; +x_25 = lean_ctor_get(x_23, 0); +lean_inc(x_25); +lean_dec(x_23); +x_26 = lean_array_size(x_25); +x_27 = 0; +lean_inc(x_25); +x_28 = l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalCase___spec__3(x_26, x_27, x_25); +x_29 = l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalCase___spec__4(x_26, x_27, x_25); +x_30 = lean_unsigned_to_nat(2u); +x_31 = l_Lean_Syntax_getArg(x_1, x_30); +x_32 = lean_unsigned_to_nat(3u); +x_33 = l_Lean_Syntax_getArg(x_1, x_32); +lean_dec(x_1); +x_34 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_addCheckpoints___spec__1___closed__4; +lean_inc(x_33); +x_35 = l_Lean_Syntax_isOfKind(x_33, x_34); +if (x_35 == 0) { -lean_object* x_35; -lean_dec(x_32); -lean_dec(x_30); +lean_object* x_36; +lean_dec(x_33); +lean_dec(x_31); +lean_dec(x_29); lean_dec(x_28); -lean_dec(x_27); +lean_dec(x_15); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -43372,20 +44031,20 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_35 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(x_10); -return x_35; +x_36 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(x_10); +return x_36; } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; size_t x_41; lean_object* x_42; -x_36 = lean_box(0); -x_37 = lean_array_get_size(x_27); -x_38 = l_Array_toSubarray___rarg(x_27, x_18, x_37); -x_39 = l_Lean_Elab_Tactic_addCheckpoints___lambda__1___closed__1; -x_40 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_40, 0, x_38); -lean_ctor_set(x_40, 1, x_39); -x_41 = lean_array_size(x_28); +lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; size_t x_42; lean_object* x_43; +x_37 = lean_box(0); +x_38 = lean_array_get_size(x_28); +x_39 = l_Array_toSubarray___rarg(x_28, x_14, x_38); +x_40 = l_Lean_Elab_Tactic_addCheckpoints___lambda__1___closed__1; +x_41 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_41, 0, x_39); +lean_ctor_set(x_41, 1, x_40); +x_42 = lean_array_size(x_29); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); @@ -43394,28 +44053,28 @@ lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); -x_42 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1(x_30, x_32, x_36, x_28, x_41, x_26, x_40, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_28); -if (lean_obj_tag(x_42) == 0) +x_43 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1(x_15, x_31, x_33, x_37, x_29, x_42, x_27, x_41, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_29); +if (lean_obj_tag(x_43) == 0) { -lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_43 = lean_ctor_get(x_42, 0); -lean_inc(x_43); -x_44 = lean_ctor_get(x_42, 1); +lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_44 = lean_ctor_get(x_43, 0); lean_inc(x_44); -lean_dec(x_42); x_45 = lean_ctor_get(x_43, 1); lean_inc(x_45); lean_dec(x_43); -x_46 = l_Lean_Elab_Tactic_getGoals___rarg(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_44); -x_47 = lean_ctor_get(x_46, 0); -lean_inc(x_47); -x_48 = lean_ctor_get(x_46, 1); +x_46 = lean_ctor_get(x_44, 1); +lean_inc(x_46); +lean_dec(x_44); +x_47 = l_Lean_Elab_Tactic_getGoals___rarg(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_45); +x_48 = lean_ctor_get(x_47, 0); lean_inc(x_48); -lean_dec(x_46); -x_49 = lean_array_to_list(x_45); -x_50 = l_List_appendTR___rarg(x_49, x_47); -x_51 = l_Lean_Elab_Tactic_setGoals(x_50, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_48); +x_49 = lean_ctor_get(x_47, 1); +lean_inc(x_49); +lean_dec(x_47); +x_50 = lean_array_to_list(x_46); +x_51 = l_List_appendTR___rarg(x_50, x_48); +x_52 = l_Lean_Elab_Tactic_setGoals(x_51, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_49); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -43424,11 +44083,11 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -return x_51; +return x_52; } else { -uint8_t x_52; +uint8_t x_53; lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -43437,23 +44096,23 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_52 = !lean_is_exclusive(x_42); -if (x_52 == 0) +x_53 = !lean_is_exclusive(x_43); +if (x_53 == 0) { -return x_42; +return x_43; } else { -lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_53 = lean_ctor_get(x_42, 0); -x_54 = lean_ctor_get(x_42, 1); +lean_object* x_54; lean_object* x_55; lean_object* x_56; +x_54 = lean_ctor_get(x_43, 0); +x_55 = lean_ctor_get(x_43, 1); +lean_inc(x_55); lean_inc(x_54); -lean_inc(x_53); -lean_dec(x_42); -x_55 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_55, 0, x_53); -lean_ctor_set(x_55, 1, x_54); -return x_55; +lean_dec(x_43); +x_56 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_56, 0, x_54); +lean_ctor_set(x_56, 1, x_55); +return x_56; } } } @@ -43479,17 +44138,34 @@ lean_dec(x_5); return x_15; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___boxed(lean_object** _args) { +lean_object* x_1 = _args[0]; +lean_object* x_2 = _args[1]; +lean_object* x_3 = _args[2]; +lean_object* x_4 = _args[3]; +lean_object* x_5 = _args[4]; +lean_object* x_6 = _args[5]; +lean_object* x_7 = _args[6]; +lean_object* x_8 = _args[7]; +lean_object* x_9 = _args[8]; +lean_object* x_10 = _args[9]; +lean_object* x_11 = _args[10]; +lean_object* x_12 = _args[11]; +lean_object* x_13 = _args[12]; +lean_object* x_14 = _args[13]; +lean_object* x_15 = _args[14]; +lean_object* x_16 = _args[15]; +lean_object* x_17 = _args[16]; _start: { -size_t x_17; size_t x_18; lean_object* x_19; -x_17 = lean_unbox_usize(x_5); -lean_dec(x_5); +size_t x_18; size_t x_19; lean_object* x_20; x_18 = lean_unbox_usize(x_6); lean_dec(x_6); -x_19 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1(x_1, x_2, x_3, x_4, x_17, x_18, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_4); -return x_19; +x_19 = lean_unbox_usize(x_7); +lean_dec(x_7); +x_20 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1(x_1, x_2, x_3, x_4, x_5, x_18, x_19, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +lean_dec(x_5); +return x_20; } } static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalCase_x27__1___closed__1() { diff --git a/stage0/stdlib/Lean/Elab/Tactic/Conv/Delta.c b/stage0/stdlib/Lean/Elab/Tactic/Conv/Delta.c index 9370452f3c42..2697ee80a9c6 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/Conv/Delta.c +++ b/stage0/stdlib/Lean/Elab/Tactic/Conv/Delta.c @@ -25,7 +25,6 @@ static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalDelta_declRange__1_ static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalDelta__1___closed__9; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Conv_evalDelta___boxed__const__1; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalDelta_declRange__1___closed__7; -lean_object* l_Array_contains___at_Lean_findField_x3f___spec__1___boxed(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalDelta_declRange__1___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalDelta__1___closed__2; lean_object* l_Lean_Elab_Tactic_Conv_changeLhs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -47,6 +46,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Conv_evalDelta(lean_object*, lean_ob static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalDelta__1___closed__5; size_t lean_array_size(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Conv_evalDelta___lambda__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_Array_contains___at_Lean_registerInternalExceptionId___spec__1___boxed(lean_object*, lean_object*); lean_object* l_Lean_Meta_deltaExpand(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalDelta__1___closed__6; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalDelta_declRange__1___closed__2; @@ -86,7 +86,7 @@ lean_inc(x_20); x_21 = lean_ctor_get(x_19, 1); lean_inc(x_21); lean_dec(x_19); -x_22 = lean_alloc_closure((void*)(l_Array_contains___at_Lean_findField_x3f___spec__1___boxed), 2, 1); +x_22 = lean_alloc_closure((void*)(l_Array_contains___at_Lean_registerInternalExceptionId___spec__1___boxed), 2, 1); lean_closure_set(x_22, 0, x_14); lean_inc(x_11); lean_inc(x_10); diff --git a/stage0/stdlib/Lean/Elab/Tactic/Conv/Pattern.c b/stage0/stdlib/Lean/Elab/Tactic/Conv/Pattern.c index cc0dadb28b5f..009ab12c4df6 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/Conv/Pattern.c +++ b/stage0/stdlib/Lean/Elab/Tactic/Conv/Pattern.c @@ -58,7 +58,6 @@ static lean_object* l___private_Lean_Elab_Tactic_Conv_Pattern_0__Lean_Elab_Tacti static lean_object* l_Lean_Elab_Tactic_Conv_evalPattern___lambda__11___closed__3; uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_stringToMessageData(lean_object*); static lean_object* l_Lean_Elab_Tactic_Conv_evalPattern___lambda__11___closed__6; LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Conv_evalPattern___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -84,6 +83,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Conv_evalPattern(lean_object*, lean_ static lean_object* l_Lean_Elab_Tactic_Conv_evalPattern___lambda__9___closed__4; lean_object* l_Lean_Elab_Term_withoutErrToSorryImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_Conv_getLhs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_forInUnsafe_loop___at_Lean_Meta_Simp_visitFn___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_qsort_sort___at_Lean_Elab_Tactic_Conv_evalPattern___spec__3___closed__1; lean_object* l_Lean_Meta_withNewMCtxDepth___at_Lean_Meta_matchesInstance___spec__1___rarg(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -91,7 +91,6 @@ lean_object* l_Lean_MessageData_ofFormat(lean_object*); lean_object* l_Lean_Elab_Tactic_Conv_getRhs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Conv_evalPattern___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Conv_matchPattern_x3f_go_x3f___closed__1; -static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__2; lean_object* l_Lean_Elab_Tactic_withMainContext___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutErrToSorry___at_Lean_Elab_Tactic_Conv_evalPattern___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static uint32_t l___private_Lean_Elab_Tactic_Conv_Pattern_0__Lean_Elab_Tactic_Conv_getContext___rarg___closed__1; @@ -118,7 +117,9 @@ static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalPattern_declRange__ LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Elab_Tactic_Conv_evalPattern___spec__9___boxed(lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_matchesNull(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Conv_evalPattern___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_appFn_x21(lean_object*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalPattern_declRange__1___closed__2; static lean_object* l_Lean_Elab_Tactic_Conv_evalPattern___lambda__9___closed__3; static lean_object* l_Lean_Elab_Tactic_Conv_evalPattern___lambda__9___closed__1; @@ -139,7 +140,6 @@ static lean_object* l_Lean_Elab_Tactic_Conv_evalPattern___closed__1; static lean_object* l_Lean_Elab_Tactic_Conv_evalPattern___lambda__11___closed__8; uint8_t lean_nat_dec_lt(lean_object*, lean_object*); uint8_t l___private_Lean_HeadIndex_0__Lean_beqHeadIndex____x40_Lean_HeadIndex___hyg_68_(lean_object*, lean_object*); -static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Conv_evalPattern___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_indentExpr(lean_object*); lean_object* l_Lean_Meta_isExprDefEqGuarded(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -147,6 +147,7 @@ static lean_object* l_Lean_Elab_Tactic_Conv_evalPattern___lambda__11___closed__7 LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Conv_evalPattern___lambda__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Conv_evalPattern___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Conv_PatternMatchState_accept(lean_object*, lean_object*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__1; LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Elab_Tactic_Conv_evalPattern___spec__3___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_isNone(lean_object*); @@ -192,7 +193,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Conv_matchPattern_x3f___lambda__1(le LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Conv_Pattern_0__Lean_Elab_Tactic_Conv_getContext___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Elab_Tactic_Conv_evalPattern___spec__3___lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalPattern__1(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_mvarId_x21(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Conv_evalPattern___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_uset(lean_object*, size_t, lean_object*); @@ -2431,7 +2431,7 @@ return x_32; } } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__1() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__1() { _start: { lean_object* x_1; @@ -2439,16 +2439,16 @@ x_1 = lean_mk_string_unchecked("positive integer expected", 25, 25); return x_1; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__2() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__1; +x_1 = l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { lean_object* x_16; uint8_t x_17; @@ -2489,7 +2489,7 @@ lean_dec(x_21); lean_dec(x_19); lean_dec(x_6); lean_dec(x_4); -x_28 = l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__2; +x_28 = l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__2; x_29 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Conv_evalPattern___spec__6(x_20, x_28, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); lean_dec(x_20); x_30 = !lean_is_exclusive(x_29); @@ -4647,7 +4647,7 @@ lean_dec(x_60); x_62 = lean_array_get_size(x_61); x_63 = lean_mk_empty_array_with_capacity(x_62); lean_inc(x_10); -x_64 = l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8(x_61, x_61, x_62, x_59, lean_box(0), x_63, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_47); +x_64 = l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8(x_61, x_61, x_62, x_59, lean_box(0), x_63, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_47); lean_dec(x_61); if (lean_obj_tag(x_64) == 0) { @@ -5049,11 +5049,11 @@ lean_dec(x_1); return x_12; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { lean_object* x_16; -x_16 = l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +x_16 = l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); lean_dec(x_14); lean_dec(x_12); lean_dec(x_11); @@ -5396,10 +5396,10 @@ l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Conv_evalPattern___spec lean_mark_persistent(l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Conv_evalPattern___spec__5___rarg___closed__1); l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Conv_evalPattern___spec__5___rarg___closed__2 = _init_l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Conv_evalPattern___spec__5___rarg___closed__2(); lean_mark_persistent(l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Conv_evalPattern___spec__5___rarg___closed__2); -l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__1 = _init_l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__1(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__1); -l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__2 = _init_l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__2(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__2); +l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__1 = _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__1(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__1); +l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__2 = _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__2(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__2); l_Lean_Elab_Tactic_Conv_evalPattern___lambda__9___closed__1 = _init_l_Lean_Elab_Tactic_Conv_evalPattern___lambda__9___closed__1(); lean_mark_persistent(l_Lean_Elab_Tactic_Conv_evalPattern___lambda__9___closed__1); l_Lean_Elab_Tactic_Conv_evalPattern___lambda__9___closed__2 = _init_l_Lean_Elab_Tactic_Conv_evalPattern___lambda__9___closed__2(); diff --git a/stage0/stdlib/Lean/Elab/Tactic/Conv/Unfold.c b/stage0/stdlib/Lean/Elab/Tactic/Conv/Unfold.c index 591d66f6584a..292cbd07556a 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/Conv/Unfold.c +++ b/stage0/stdlib/Lean/Elab/Tactic/Conv/Unfold.c @@ -13,66 +13,79 @@ #ifdef __cplusplus extern "C" { #endif +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Conv_evalUnfold___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_KeyedDeclsAttribute_addBuiltin___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3___closed__1; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___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_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Conv_evalUnfold___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_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___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*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Conv_evalUnfold___lambda__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3___closed__3; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalUnfold_declRange__1___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalUnfold_declRange__1___closed__7; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__2; extern lean_object* l_Lean_Elab_Tactic_tacticElabAttribute; lean_object* l_Lean_Meta_unfold(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalUnfold__1___closed__6; +lean_object* l_Lean_FVarId_isLetVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getArgs(lean_object*); lean_object* l_Lean_replaceRef(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalUnfold__1(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalUnfold__1___closed__8; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__7; lean_object* l_Lean_addBuiltinDeclarationRanges(lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalUnfold__1___closed__5; -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Conv_evalUnfold___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_Name_mkStr5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Conv_evalUnfold___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_stringToMessageData(lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3___closed__4; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Conv_evalUnfold___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t l_Lean_Expr_hasMVar(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Conv_evalUnfold(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__1___closed__1; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___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_st_ref_take(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalUnfold_declRange__1(lean_object*); lean_object* l_Lean_Elab_Tactic_Conv_changeLhs(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*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalUnfold_declRange__1___closed__5; -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3___closed__5; lean_object* l_Lean_Elab_Tactic_withMainContext___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_zetaDeltaFVars(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_Conv_evalUnfold___spec__3___closed__2; +lean_object* lean_st_ref_get(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Conv_evalUnfold___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_Tactic_elabTermForApply(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_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_instantiateMVars___at_Lean_Elab_Tactic_Conv_evalUnfold___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_instantiateMVars___at_Lean_Elab_Tactic_Conv_evalUnfold___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_Lean_Elab_Tactic_Conv_evalUnfold___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*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalUnfold_declRange__1___closed__6; lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalUnfold__1___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalUnfold_declRange__1___closed__2; lean_object* l_Lean_MessageData_ofExpr(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*); -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Conv_evalUnfold___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_evalUnfold_declRange__1___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalUnfold__1___closed__11; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalUnfold__1___closed__10; -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalUnfold__1___closed__3; lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalUnfold__1___closed__9; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalUnfold__1___closed__2; lean_object* lean_array_mk(lean_object*); +lean_object* l_Lean_instantiateMVarsCore(lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Conv_evalUnfold___boxed__const__1; lean_object* lean_array_uget(lean_object*, size_t); +lean_object* l_Lean_Expr_fvar___override(lean_object*); size_t lean_array_size(lean_object*); +lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__8; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalUnfold__1___closed__1; -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); lean_object* l_Lean_Elab_Tactic_Conv_applySimpResult(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__1___closed__7; -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Conv_evalUnfold___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) { +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__5; +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Conv_evalUnfold___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; @@ -110,93 +123,341 @@ return x_19; } } } -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Conv_evalUnfold___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_instantiateMVars___at_Lean_Elab_Tactic_Conv_evalUnfold___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: { -uint8_t x_12; -x_12 = !lean_is_exclusive(x_9); -if (x_12 == 0) +uint8_t x_11; +x_11 = l_Lean_Expr_hasMVar(x_1); +if (x_11 == 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_object* x_12; +x_12 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_1); +lean_ctor_set(x_12, 1, x_10); +return x_12; +} +else +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_13 = lean_st_ref_get(x_7, x_10); +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_13, 1); +lean_inc(x_15); lean_dec(x_13); -lean_ctor_set(x_9, 5, x_14); -x_15 = l_Lean_throwError___at_Lean_Elab_Tactic_Conv_evalUnfold___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_9); -return x_15; +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_take(x_7, x_15); +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +x_23 = !lean_is_exclusive(x_21); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; uint8_t x_26; +x_24 = lean_ctor_get(x_21, 0); +lean_dec(x_24); +lean_ctor_set(x_21, 0, x_19); +x_25 = lean_st_ref_set(x_7, x_21, x_22); +x_26 = !lean_is_exclusive(x_25); +if (x_26 == 0) +{ +lean_object* x_27; +x_27 = lean_ctor_get(x_25, 0); +lean_dec(x_27); +lean_ctor_set(x_25, 0, x_18); +return x_25; } else { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; lean_object* x_28; uint8_t x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; -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); -x_27 = lean_ctor_get_uint8(x_9, sizeof(void*)*12); -x_28 = lean_ctor_get(x_9, 11); -x_29 = lean_ctor_get_uint8(x_9, sizeof(void*)*12 + 1); +lean_object* x_28; lean_object* x_29; +x_28 = lean_ctor_get(x_25, 1); lean_inc(x_28); -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_dec(x_25); +x_29 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_29, 0, x_18); +lean_ctor_set(x_29, 1, x_28); +return x_29; +} +} +else +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_30 = lean_ctor_get(x_21, 1); +x_31 = lean_ctor_get(x_21, 2); +x_32 = lean_ctor_get(x_21, 3); +x_33 = lean_ctor_get(x_21, 4); +lean_inc(x_33); +lean_inc(x_32); +lean_inc(x_31); +lean_inc(x_30); +lean_dec(x_21); +x_34 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_34, 0, x_19); +lean_ctor_set(x_34, 1, x_30); +lean_ctor_set(x_34, 2, x_31); +lean_ctor_set(x_34, 3, x_32); +lean_ctor_set(x_34, 4, x_33); +x_35 = lean_st_ref_set(x_7, x_34, x_22); +x_36 = lean_ctor_get(x_35, 1); +lean_inc(x_36); +if (lean_is_exclusive(x_35)) { + lean_ctor_release(x_35, 0); + lean_ctor_release(x_35, 1); + x_37 = x_35; +} else { + lean_dec_ref(x_35); + x_37 = lean_box(0); +} +if (lean_is_scalar(x_37)) { + x_38 = lean_alloc_ctor(0, 2, 0); +} else { + x_38 = x_37; +} +lean_ctor_set(x_38, 0, x_18); +lean_ctor_set(x_38, 1, x_36); +return x_38; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; 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_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +x_12 = l_Lean_Elab_Tactic_Conv_getLhs(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; uint8_t x_16; +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_12, 1); +lean_inc(x_14); +lean_dec(x_12); +x_15 = l_Lean_instantiateMVars___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__2(x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_14); +x_16 = !lean_is_exclusive(x_15); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_17 = lean_ctor_get(x_15, 0); +x_18 = lean_ctor_get(x_15, 1); +x_19 = lean_box(0); +lean_ctor_set_tag(x_15, 1); +lean_ctor_set(x_15, 1, x_19); +lean_ctor_set(x_15, 0, x_1); +x_20 = lean_array_mk(x_15); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +x_21 = l_Lean_Meta_zetaDeltaFVars(x_17, x_20, x_7, x_8, x_9, x_10, x_18); +if (lean_obj_tag(x_21) == 0) +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_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_Elab_Tactic_Conv_changeLhs(x_22, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_23); +return x_24; +} +else +{ +uint8_t x_25; +lean_dec(x_10); lean_dec(x_9); -x_30 = l_Lean_replaceRef(x_1, x_21); +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_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_31 = lean_alloc_ctor(0, 12, 2); -lean_ctor_set(x_31, 0, x_16); -lean_ctor_set(x_31, 1, x_17); -lean_ctor_set(x_31, 2, x_18); -lean_ctor_set(x_31, 3, x_19); -lean_ctor_set(x_31, 4, x_20); -lean_ctor_set(x_31, 5, x_30); -lean_ctor_set(x_31, 6, x_22); -lean_ctor_set(x_31, 7, x_23); -lean_ctor_set(x_31, 8, x_24); -lean_ctor_set(x_31, 9, x_25); -lean_ctor_set(x_31, 10, x_26); -lean_ctor_set(x_31, 11, x_28); -lean_ctor_set_uint8(x_31, sizeof(void*)*12, x_27); -lean_ctor_set_uint8(x_31, sizeof(void*)*12 + 1, x_29); -x_32 = l_Lean_throwError___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__2(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_31, x_10, x_11); -lean_dec(x_31); -return x_32; -} -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3___closed__1() { +x_28 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +return x_28; +} +} +} +else +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_29 = lean_ctor_get(x_15, 0); +x_30 = lean_ctor_get(x_15, 1); +lean_inc(x_30); +lean_inc(x_29); +lean_dec(x_15); +x_31 = lean_box(0); +x_32 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_32, 0, x_1); +lean_ctor_set(x_32, 1, x_31); +x_33 = lean_array_mk(x_32); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +x_34 = l_Lean_Meta_zetaDeltaFVars(x_29, x_33, x_7, x_8, x_9, x_10, x_30); +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); +x_37 = l_Lean_Elab_Tactic_Conv_changeLhs(x_35, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_36); +return x_37; +} +else +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_38 = lean_ctor_get(x_34, 0); +lean_inc(x_38); +x_39 = lean_ctor_get(x_34, 1); +lean_inc(x_39); +if (lean_is_exclusive(x_34)) { + lean_ctor_release(x_34, 0); + lean_ctor_release(x_34, 1); + x_40 = x_34; +} else { + lean_dec_ref(x_34); + x_40 = lean_box(0); +} +if (lean_is_scalar(x_40)) { + x_41 = lean_alloc_ctor(1, 2, 0); +} else { + x_41 = x_40; +} +lean_ctor_set(x_41, 0, x_38); +lean_ctor_set(x_41, 1, x_39); +return x_41; +} +} +} +else +{ +uint8_t x_42; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_42 = !lean_is_exclusive(x_12); +if (x_42 == 0) +{ +return x_12; +} +else +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_12, 0); +x_44 = lean_ctor_get(x_12, 1); +lean_inc(x_44); +lean_inc(x_43); +lean_dec(x_12); +x_45 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_45, 0, x_43); +lean_ctor_set(x_45, 1, x_44); +return x_45; +} +} +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("'unfold' conv tactic failed, expression ", 40, 40); +x_1 = lean_mk_string_unchecked("conv tactic 'unfold' failed, expression ", 40, 40); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3___closed__2() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3___closed__1; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3___closed__3() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__3() { _start: { lean_object* x_1; @@ -204,26 +465,50 @@ x_1 = lean_mk_string_unchecked(" is not a global or local constant", 34, 34); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3___closed__4() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("conv tactic 'unfold' failed, local variable '", 45, 45); +return x_1; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__6() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3___closed__3; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__5; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3___closed__5() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__7() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("' has no definition", 19, 19); +return x_1; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__8() { _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); +x_1 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__7; +x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___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) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___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, lean_object* x_12, lean_object* x_13) { _start: { uint8_t x_14; @@ -232,7 +517,6 @@ if (x_14 == 0) { lean_object* x_15; lean_dec(x_12); -lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -246,539 +530,361 @@ return x_15; } else { -lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_24; lean_object* x_25; +lean_object* x_16; lean_object* x_17; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; 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; uint8_t x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; lean_object* x_45; lean_dec(x_4); x_16 = lean_array_uget(x_1, x_3); -x_24 = 0; +x_28 = lean_ctor_get(x_11, 0); +x_29 = lean_ctor_get(x_11, 1); +x_30 = lean_ctor_get(x_11, 2); +x_31 = lean_ctor_get(x_11, 3); +x_32 = lean_ctor_get(x_11, 4); +x_33 = lean_ctor_get(x_11, 5); +x_34 = lean_ctor_get(x_11, 6); +x_35 = lean_ctor_get(x_11, 7); +x_36 = lean_ctor_get(x_11, 8); +x_37 = lean_ctor_get(x_11, 9); +x_38 = lean_ctor_get(x_11, 10); +x_39 = lean_ctor_get_uint8(x_11, sizeof(void*)*12); +x_40 = lean_ctor_get(x_11, 11); +x_41 = lean_ctor_get_uint8(x_11, sizeof(void*)*12 + 1); +x_42 = l_Lean_replaceRef(x_16, x_33); +lean_inc(x_40); +lean_inc(x_38); +lean_inc(x_37); +lean_inc(x_36); +lean_inc(x_35); +lean_inc(x_34); +lean_inc(x_32); +lean_inc(x_31); +lean_inc(x_30); +lean_inc(x_29); +lean_inc(x_28); +x_43 = lean_alloc_ctor(0, 12, 2); +lean_ctor_set(x_43, 0, x_28); +lean_ctor_set(x_43, 1, x_29); +lean_ctor_set(x_43, 2, x_30); +lean_ctor_set(x_43, 3, x_31); +lean_ctor_set(x_43, 4, x_32); +lean_ctor_set(x_43, 5, x_42); +lean_ctor_set(x_43, 6, x_34); +lean_ctor_set(x_43, 7, x_35); +lean_ctor_set(x_43, 8, x_36); +lean_ctor_set(x_43, 9, x_37); +lean_ctor_set(x_43, 10, x_38); +lean_ctor_set(x_43, 11, x_40); +lean_ctor_set_uint8(x_43, sizeof(void*)*12, x_39); +lean_ctor_set_uint8(x_43, sizeof(void*)*12 + 1, x_41); +x_44 = 0; lean_inc(x_12); -lean_inc(x_11); +lean_inc(x_43); 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_16); -x_25 = l_Lean_Elab_Tactic_elabTermForApply(x_16, x_24, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_25) == 0) +x_45 = l_Lean_Elab_Tactic_elabTermForApply(x_16, x_44, x_5, x_6, x_7, x_8, x_9, x_10, x_43, x_12, x_13); +if (lean_obj_tag(x_45) == 0) { -lean_object* x_26; -x_26 = lean_ctor_get(x_25, 0); -lean_inc(x_26); -switch (lean_obj_tag(x_26)) { +lean_object* x_46; +x_46 = lean_ctor_get(x_45, 0); +lean_inc(x_46); +switch (lean_obj_tag(x_46)) { case 1: { -lean_object* x_27; lean_object* x_28; lean_object* x_29; -lean_dec(x_16); -x_27 = lean_ctor_get(x_25, 1); -lean_inc(x_27); -lean_dec(x_25); -x_28 = lean_ctor_get(x_26, 0); -lean_inc(x_28); -lean_dec(x_26); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -x_29 = l_Lean_Elab_Tactic_Conv_getLhs(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_27); -if (lean_obj_tag(x_29) == 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); -x_32 = l_Lean_instantiateMVars___at_Lean_Elab_Tactic_getMainTarget___spec__1(x_30, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_31); -x_33 = !lean_is_exclusive(x_32); -if (x_33 == 0) -{ -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_34 = lean_ctor_get(x_32, 0); -x_35 = lean_ctor_get(x_32, 1); -x_36 = lean_box(0); -lean_ctor_set_tag(x_32, 1); -lean_ctor_set(x_32, 1, x_36); -lean_ctor_set(x_32, 0, x_28); -x_37 = lean_array_mk(x_32); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -x_38 = l_Lean_Meta_zetaDeltaFVars(x_34, x_37, x_9, x_10, x_11, x_12, x_35); -if (lean_obj_tag(x_38) == 0) -{ -lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_39 = lean_ctor_get(x_38, 0); -lean_inc(x_39); -x_40 = lean_ctor_get(x_38, 1); -lean_inc(x_40); -lean_dec(x_38); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); +lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_47 = lean_ctor_get(x_45, 1); +lean_inc(x_47); +lean_dec(x_45); +x_48 = lean_ctor_get(x_46, 0); +lean_inc(x_48); +lean_dec(x_46); lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -x_41 = l_Lean_Elab_Tactic_Conv_changeLhs(x_39, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_40); -if (lean_obj_tag(x_41) == 0) -{ -lean_object* x_42; lean_object* x_43; -x_42 = lean_ctor_get(x_41, 1); -lean_inc(x_42); -lean_dec(x_41); -x_43 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3___closed__5; -x_17 = x_43; -x_18 = x_42; -goto block_23; -} -else -{ -uint8_t x_44; -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -x_44 = !lean_is_exclusive(x_41); -if (x_44 == 0) -{ -return x_41; -} -else -{ -lean_object* x_45; lean_object* x_46; lean_object* x_47; -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_alloc_ctor(1, 2, 0); -lean_ctor_set(x_47, 0, x_45); -lean_ctor_set(x_47, 1, x_46); -return x_47; -} -} -} -else +lean_inc(x_48); +x_49 = l_Lean_FVarId_isLetVar(x_48, x_9, x_10, x_43, x_12, x_47); +if (lean_obj_tag(x_49) == 0) { -uint8_t x_48; -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -x_48 = !lean_is_exclusive(x_38); -if (x_48 == 0) +lean_object* x_50; uint8_t x_51; +x_50 = lean_ctor_get(x_49, 0); +lean_inc(x_50); +x_51 = lean_unbox(x_50); +lean_dec(x_50); +if (x_51 == 0) { -return x_38; +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_52 = lean_ctor_get(x_49, 1); +lean_inc(x_52); +lean_dec(x_49); +x_53 = l_Lean_Expr_fvar___override(x_48); +x_54 = l_Lean_MessageData_ofExpr(x_53); +x_55 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__6; +x_56 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_56, 0, x_55); +lean_ctor_set(x_56, 1, x_54); +x_57 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__8; +x_58 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_58, 0, x_56); +lean_ctor_set(x_58, 1, x_57); +x_59 = l_Lean_throwError___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3(x_58, x_5, x_6, x_7, x_8, x_9, x_10, x_43, x_12, x_52); +lean_dec(x_43); +x_60 = !lean_is_exclusive(x_59); +if (x_60 == 0) +{ +x_17 = x_59; +goto block_27; } else { -lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_49 = lean_ctor_get(x_38, 0); -x_50 = lean_ctor_get(x_38, 1); -lean_inc(x_50); -lean_inc(x_49); -lean_dec(x_38); -x_51 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_51, 0, x_49); -lean_ctor_set(x_51, 1, x_50); -return x_51; -} +lean_object* x_61; lean_object* x_62; lean_object* x_63; +x_61 = lean_ctor_get(x_59, 0); +x_62 = lean_ctor_get(x_59, 1); +lean_inc(x_62); +lean_inc(x_61); +lean_dec(x_59); +x_63 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_63, 0, x_61); +lean_ctor_set(x_63, 1, x_62); +x_17 = x_63; +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; -x_52 = lean_ctor_get(x_32, 0); -x_53 = lean_ctor_get(x_32, 1); -lean_inc(x_53); -lean_inc(x_52); -lean_dec(x_32); -x_54 = lean_box(0); -x_55 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_55, 0, x_28); -lean_ctor_set(x_55, 1, x_54); -x_56 = lean_array_mk(x_55); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -x_57 = l_Lean_Meta_zetaDeltaFVars(x_52, x_56, x_9, x_10, x_11, x_12, x_53); -if (lean_obj_tag(x_57) == 0) -{ -lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_58 = lean_ctor_get(x_57, 0); -lean_inc(x_58); -x_59 = lean_ctor_get(x_57, 1); -lean_inc(x_59); -lean_dec(x_57); +lean_object* x_64; lean_object* x_65; lean_object* x_66; +x_64 = lean_ctor_get(x_49, 1); +lean_inc(x_64); +lean_dec(x_49); +x_65 = 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); lean_inc(x_6); lean_inc(x_5); -x_60 = l_Lean_Elab_Tactic_Conv_changeLhs(x_58, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_59); -if (lean_obj_tag(x_60) == 0) -{ -lean_object* x_61; lean_object* x_62; -x_61 = lean_ctor_get(x_60, 1); -lean_inc(x_61); -lean_dec(x_60); -x_62 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3___closed__5; -x_17 = x_62; -x_18 = x_61; -goto block_23; -} -else -{ -lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -x_63 = lean_ctor_get(x_60, 0); -lean_inc(x_63); -x_64 = lean_ctor_get(x_60, 1); -lean_inc(x_64); -if (lean_is_exclusive(x_60)) { - lean_ctor_release(x_60, 0); - lean_ctor_release(x_60, 1); - x_65 = x_60; -} else { - lean_dec_ref(x_60); - x_65 = lean_box(0); -} -if (lean_is_scalar(x_65)) { - x_66 = lean_alloc_ctor(1, 2, 0); -} else { - x_66 = x_65; -} -lean_ctor_set(x_66, 0, x_63); -lean_ctor_set(x_66, 1, x_64); -return x_66; -} -} -else -{ -lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -x_67 = lean_ctor_get(x_57, 0); -lean_inc(x_67); -x_68 = lean_ctor_get(x_57, 1); -lean_inc(x_68); -if (lean_is_exclusive(x_57)) { - lean_ctor_release(x_57, 0); - lean_ctor_release(x_57, 1); - x_69 = x_57; -} else { - lean_dec_ref(x_57); - x_69 = lean_box(0); -} -if (lean_is_scalar(x_69)) { - x_70 = lean_alloc_ctor(1, 2, 0); -} else { - x_70 = x_69; -} -lean_ctor_set(x_70, 0, x_67); -lean_ctor_set(x_70, 1, x_68); -return x_70; -} +x_66 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___lambda__1(x_48, x_65, x_5, x_6, x_7, x_8, x_9, x_10, x_43, x_12, x_64); +x_17 = x_66; +goto block_27; } } else { -uint8_t x_71; -lean_dec(x_28); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -x_71 = !lean_is_exclusive(x_29); -if (x_71 == 0) +uint8_t x_67; +lean_dec(x_48); +lean_dec(x_43); +x_67 = !lean_is_exclusive(x_49); +if (x_67 == 0) { -return x_29; +x_17 = x_49; +goto block_27; } else { -lean_object* x_72; lean_object* x_73; lean_object* x_74; -x_72 = lean_ctor_get(x_29, 0); -x_73 = lean_ctor_get(x_29, 1); -lean_inc(x_73); -lean_inc(x_72); -lean_dec(x_29); -x_74 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_74, 0, x_72); -lean_ctor_set(x_74, 1, x_73); -return x_74; +lean_object* x_68; lean_object* x_69; lean_object* x_70; +x_68 = lean_ctor_get(x_49, 0); +x_69 = lean_ctor_get(x_49, 1); +lean_inc(x_69); +lean_inc(x_68); +lean_dec(x_49); +x_70 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_70, 0, x_68); +lean_ctor_set(x_70, 1, x_69); +x_17 = x_70; +goto block_27; } } } case 4: { -lean_object* x_75; lean_object* x_76; lean_object* x_77; -lean_dec(x_16); -x_75 = lean_ctor_get(x_25, 1); -lean_inc(x_75); -lean_dec(x_25); -x_76 = lean_ctor_get(x_26, 0); -lean_inc(x_76); -lean_dec(x_26); +lean_object* x_71; lean_object* x_72; lean_object* x_73; +x_71 = lean_ctor_get(x_45, 1); +lean_inc(x_71); +lean_dec(x_45); +x_72 = lean_ctor_get(x_46, 0); +lean_inc(x_72); +lean_dec(x_46); lean_inc(x_12); -lean_inc(x_11); +lean_inc(x_43); lean_inc(x_10); lean_inc(x_9); -x_77 = l_Lean_Elab_Tactic_Conv_getLhs(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_75); -if (lean_obj_tag(x_77) == 0) +x_73 = l_Lean_Elab_Tactic_Conv_getLhs(x_5, x_6, x_7, x_8, x_9, x_10, x_43, x_12, x_71); +if (lean_obj_tag(x_73) == 0) { -lean_object* x_78; lean_object* x_79; lean_object* x_80; -x_78 = lean_ctor_get(x_77, 0); -lean_inc(x_78); -x_79 = lean_ctor_get(x_77, 1); -lean_inc(x_79); -lean_dec(x_77); +lean_object* x_74; lean_object* x_75; lean_object* 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); lean_inc(x_12); -lean_inc(x_11); +lean_inc(x_43); lean_inc(x_10); lean_inc(x_9); -x_80 = l_Lean_Meta_unfold(x_78, x_76, x_9, x_10, x_11, x_12, x_79); -if (lean_obj_tag(x_80) == 0) +x_76 = l_Lean_Meta_unfold(x_74, x_72, x_9, x_10, x_43, x_12, x_75); +if (lean_obj_tag(x_76) == 0) { -lean_object* x_81; lean_object* x_82; lean_object* x_83; -x_81 = lean_ctor_get(x_80, 0); -lean_inc(x_81); -x_82 = lean_ctor_get(x_80, 1); -lean_inc(x_82); -lean_dec(x_80); +lean_object* x_77; lean_object* x_78; lean_object* x_79; +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_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_83 = l_Lean_Elab_Tactic_Conv_applySimpResult(x_81, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_82); -if (lean_obj_tag(x_83) == 0) -{ -lean_object* x_84; lean_object* x_85; -x_84 = lean_ctor_get(x_83, 1); -lean_inc(x_84); -lean_dec(x_83); -x_85 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3___closed__5; -x_17 = x_85; -x_18 = x_84; -goto block_23; +x_79 = l_Lean_Elab_Tactic_Conv_applySimpResult(x_77, x_5, x_6, x_7, x_8, x_9, x_10, x_43, x_12, x_78); +x_17 = x_79; +goto block_27; } else { -uint8_t x_86; -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -x_86 = !lean_is_exclusive(x_83); -if (x_86 == 0) +uint8_t x_80; +lean_dec(x_43); +x_80 = !lean_is_exclusive(x_76); +if (x_80 == 0) { -return x_83; +x_17 = x_76; +goto block_27; } else { -lean_object* x_87; lean_object* x_88; lean_object* x_89; -x_87 = lean_ctor_get(x_83, 0); -x_88 = lean_ctor_get(x_83, 1); -lean_inc(x_88); -lean_inc(x_87); -lean_dec(x_83); -x_89 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_89, 0, x_87); -lean_ctor_set(x_89, 1, x_88); -return x_89; +lean_object* x_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_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); +x_17 = x_83; +goto block_27; } } } else { -uint8_t x_90; -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -x_90 = !lean_is_exclusive(x_80); -if (x_90 == 0) +uint8_t x_84; +lean_dec(x_72); +lean_dec(x_43); +x_84 = !lean_is_exclusive(x_73); +if (x_84 == 0) { -return x_80; +x_17 = x_73; +goto block_27; } else { -lean_object* x_91; lean_object* x_92; lean_object* x_93; -x_91 = lean_ctor_get(x_80, 0); -x_92 = lean_ctor_get(x_80, 1); -lean_inc(x_92); -lean_inc(x_91); -lean_dec(x_80); -x_93 = lean_alloc_ctor(1, 2, 0); +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_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); +x_17 = x_87; +goto block_27; +} +} +} +default: +{ +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_88 = lean_ctor_get(x_45, 1); +lean_inc(x_88); +lean_dec(x_45); +x_89 = l_Lean_MessageData_ofExpr(x_46); +x_90 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__2; +x_91 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_91, 0, x_90); +lean_ctor_set(x_91, 1, x_89); +x_92 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__4; +x_93 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_93, 0, x_91); lean_ctor_set(x_93, 1, x_92); -return x_93; +x_94 = l_Lean_throwError___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__1(x_93, x_5, x_6, x_7, x_8, x_9, x_10, x_43, x_12, x_88); +lean_dec(x_43); +x_17 = x_94; +goto block_27; } } } else { -uint8_t x_94; -lean_dec(x_76); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -x_94 = !lean_is_exclusive(x_77); -if (x_94 == 0) +uint8_t x_95; +lean_dec(x_43); +x_95 = !lean_is_exclusive(x_45); +if (x_95 == 0) { -return x_77; +x_17 = x_45; +goto block_27; } else { -lean_object* x_95; lean_object* x_96; lean_object* x_97; -x_95 = lean_ctor_get(x_77, 0); -x_96 = lean_ctor_get(x_77, 1); +lean_object* x_96; lean_object* x_97; lean_object* x_98; +x_96 = lean_ctor_get(x_45, 0); +x_97 = lean_ctor_get(x_45, 1); +lean_inc(x_97); lean_inc(x_96); -lean_inc(x_95); -lean_dec(x_77); -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_dec(x_45); +x_98 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_98, 0, x_96); +lean_ctor_set(x_98, 1, x_97); +x_17 = x_98; +goto block_27; } } -default: -{ -lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; uint8_t x_105; -x_98 = lean_ctor_get(x_25, 1); -lean_inc(x_98); -lean_dec(x_25); -x_99 = l_Lean_MessageData_ofExpr(x_26); -x_100 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3___closed__2; -x_101 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_101, 0, x_100); -lean_ctor_set(x_101, 1, x_99); -x_102 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3___closed__4; -x_103 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_103, 0, x_101); -lean_ctor_set(x_103, 1, x_102); -x_104 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__1(x_16, x_103, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_98); -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_16); -x_105 = !lean_is_exclusive(x_104); -if (x_105 == 0) +block_27: { -return x_104; -} -else +if (lean_obj_tag(x_17) == 0) { -lean_object* x_106; lean_object* x_107; lean_object* x_108; -x_106 = lean_ctor_get(x_104, 0); -x_107 = lean_ctor_get(x_104, 1); -lean_inc(x_107); -lean_inc(x_106); -lean_dec(x_104); -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; -} -} -} +lean_object* x_18; size_t x_19; size_t x_20; lean_object* x_21; +x_18 = lean_ctor_get(x_17, 1); +lean_inc(x_18); +lean_dec(x_17); +x_19 = 1; +x_20 = lean_usize_add(x_3, x_19); +x_21 = lean_box(0); +x_3 = x_20; +x_4 = x_21; +x_13 = x_18; +goto _start; } else { -uint8_t x_109; -lean_dec(x_16); +uint8_t x_23; lean_dec(x_12); -lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -x_109 = !lean_is_exclusive(x_25); -if (x_109 == 0) +x_23 = !lean_is_exclusive(x_17); +if (x_23 == 0) { -return x_25; +return x_17; } else { -lean_object* x_110; lean_object* x_111; lean_object* x_112; -x_110 = lean_ctor_get(x_25, 0); -x_111 = lean_ctor_get(x_25, 1); -lean_inc(x_111); -lean_inc(x_110); -lean_dec(x_25); -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_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_17, 0); +x_25 = lean_ctor_get(x_17, 1); +lean_inc(x_25); +lean_inc(x_24); +lean_dec(x_17); +x_26 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_26, 0, x_24); +lean_ctor_set(x_26, 1, x_25); +return x_26; } } -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_3, x_20); -x_3 = x_21; -x_4 = x_19; -x_13 = x_18; -goto _start; } } } @@ -788,7 +894,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Conv_evalUnfold___lambda__1(lean_obj { lean_object* x_13; lean_object* x_14; x_13 = lean_box(0); -x_14 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3(x_1, x_2, x_3, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_14 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4(x_1, x_2, x_3, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); if (lean_obj_tag(x_14) == 0) { uint8_t x_15; @@ -865,11 +971,11 @@ x_18 = l_Lean_Elab_Tactic_withMainContext___rarg(x_17, x_2, x_3, x_4, x_5, x_6, return x_18; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Conv_evalUnfold___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_throwError___at_Lean_Elab_Tactic_Conv_evalUnfold___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_Conv_evalUnfold___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_throwError___at_Lean_Elab_Tactic_Conv_evalUnfold___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); @@ -881,23 +987,48 @@ lean_dec(x_2); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Tactic_Conv_evalUnfold___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_12; -x_12 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Conv_evalUnfold___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_object* x_11; +x_11 = l_Lean_instantiateMVars___at_Lean_Elab_Tactic_Conv_evalUnfold___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_1); +lean_dec(x_2); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_throwError___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___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) { +_start: +{ +lean_object* x_12; +x_12 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___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); +lean_dec(x_2); return x_12; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { size_t x_14; size_t x_15; lean_object* x_16; @@ -905,7 +1036,8 @@ 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_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___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); +x_16 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4(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_11); lean_dec(x_1); return x_16; } @@ -919,6 +1051,7 @@ lean_dec(x_2); x_14 = lean_unbox_usize(x_3); lean_dec(x_3); x_15 = l_Lean_Elab_Tactic_Conv_evalUnfold___lambda__1(x_1, x_13, x_14, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_10); lean_dec(x_1); return x_15; } @@ -1157,16 +1290,22 @@ lean_dec_ref(res); res = initialize_Lean_Elab_Tactic_Conv_Simp(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3___closed__1); -l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3___closed__2 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3___closed__2(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3___closed__2); -l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3___closed__3 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3___closed__3(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3___closed__3); -l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3___closed__4 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3___closed__4(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3___closed__4); -l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3___closed__5 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3___closed__5(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__3___closed__5); +l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__1(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__1); +l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__2 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__2(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__2); +l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__3 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__3(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__3); +l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__4 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__4(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__4); +l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__5 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__5(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__5); +l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__6 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__6(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__6); +l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__7 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__7(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__7); +l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__8 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__8(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Conv_evalUnfold___spec__4___closed__8); l_Lean_Elab_Tactic_Conv_evalUnfold___boxed__const__1 = _init_l_Lean_Elab_Tactic_Conv_evalUnfold___boxed__const__1(); lean_mark_persistent(l_Lean_Elab_Tactic_Conv_evalUnfold___boxed__const__1); l___regBuiltin_Lean_Elab_Tactic_Conv_evalUnfold__1___closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalUnfold__1___closed__1(); diff --git a/stage0/stdlib/Lean/Elab/Tactic/Delta.c b/stage0/stdlib/Lean/Elab/Tactic/Delta.c index 084d7fb2b395..4a33b8271fb6 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/Delta.c +++ b/stage0/stdlib/Lean/Elab/Tactic/Delta.c @@ -40,7 +40,6 @@ static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalDelta__1___closed__9; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_deltaLocalDecl___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_evalDelta___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_Tactic_withLocation(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Array_contains___at_Lean_findField_x3f___spec__1___boxed(lean_object*, lean_object*); uint8_t lean_expr_eqv(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_deltaLocalDecl___closed__8; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalDelta_declRange__1___closed__2; @@ -78,6 +77,7 @@ lean_object* l_Lean_MVarId_replaceLocalDeclDefEq(lean_object*, lean_object*, lea static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalDelta__1___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_deltaTarget___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); +lean_object* l_Array_contains___at_Lean_registerInternalExceptionId___spec__1___boxed(lean_object*, lean_object*); lean_object* l_List_mapTR_loop___at_Lean_compileDecl___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalDelta(lean_object*, 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_deltaLocalDecl___closed__5; @@ -239,7 +239,7 @@ lean_inc(x_17); lean_dec(x_15); x_18 = l_Lean_LocalDecl_type(x_16); lean_inc(x_1); -x_19 = lean_alloc_closure((void*)(l_Array_contains___at_Lean_findField_x3f___spec__1___boxed), 2, 1); +x_19 = lean_alloc_closure((void*)(l_Array_contains___at_Lean_registerInternalExceptionId___spec__1___boxed), 2, 1); lean_closure_set(x_19, 0, x_1); lean_inc(x_10); lean_inc(x_9); @@ -515,7 +515,7 @@ x_16 = lean_ctor_get(x_14, 1); lean_inc(x_16); lean_dec(x_14); lean_inc(x_1); -x_17 = lean_alloc_closure((void*)(l_Array_contains___at_Lean_findField_x3f___spec__1___boxed), 2, 1); +x_17 = lean_alloc_closure((void*)(l_Array_contains___at_Lean_registerInternalExceptionId___spec__1___boxed), 2, 1); lean_closure_set(x_17, 0, x_1); lean_inc(x_9); lean_inc(x_8); diff --git a/stage0/stdlib/Lean/Elab/Tactic/Doc.c b/stage0/stdlib/Lean/Elab/Tactic/Doc.c index 43bfd1d6e576..a0328f25ea96 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/Doc.c +++ b/stage0/stdlib/Lean/Elab/Tactic/Doc.c @@ -205,7 +205,6 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Doc_allT LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Doc_elabPrintTacTags___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Doc_elabRegisterTacticTag___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Doc_allTacticDocs___lambda__3(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_Command_expandDeclId___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Tactic_Doc_0__Lean_Elab_Tactic_Doc_getFirstTk___closed__14; static lean_object* l___private_Lean_Elab_Tactic_Doc_0__Lean_Elab_Tactic_Doc_getFirstTk___closed__17; extern lean_object* l_Lean_Parser_Tactic_Doc_tacticTagExt; @@ -285,6 +284,7 @@ uint8_t lean_nat_dec_le(lean_object*, lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); lean_object* l_Lean_RBNode_find___at_Lean_NameMap_find_x3f___spec__1___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Doc_elabTacticExtension___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_throwError___at_Lean_withSetOptionIn___spec__7(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); static lean_object* l_List_mapM_loop___at_Lean_Elab_Tactic_Doc_elabPrintTacTags___spec__9___closed__1; static lean_object* l_Lean_Elab_Tactic_Doc_allTacticDocs___closed__2; @@ -320,7 +320,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_expandDeclId___spec__4(x_2, x_3, x_4, x_8); +x_12 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__7(x_2, x_3, x_4, x_8); return x_12; } else @@ -358,7 +358,7 @@ lean_ctor_set(x_23, 7, x_19); lean_ctor_set(x_23, 8, x_20); lean_ctor_set(x_23, 9, x_21); lean_ctor_set_uint8(x_23, sizeof(void*)*10, x_22); -x_24 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_2, x_23, x_4, x_8); +x_24 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__7(x_2, x_23, x_4, x_8); return x_24; } } diff --git a/stage0/stdlib/Lean/Elab/Tactic/ElabTerm.c b/stage0/stdlib/Lean/Elab/Tactic/ElabTerm.c index f14243ed7cd2..d006d8195a0d 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/ElabTerm.c +++ b/stage0/stdlib/Lean/Elab/Tactic/ElabTerm.c @@ -128,7 +128,6 @@ lean_object* l_Lean_Name_lt___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_withCollectingNewGoalsFrom_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* l_Array_qpartition___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalNativeDecide__1___closed__1; -uint8_t l_Array_contains___at_Lean_findField_x3f___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___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_evalDecideCore_diagnose___lambda__4___closed__53; lean_object* lean_mk_array(lean_object*, lean_object*); @@ -550,6 +549,7 @@ static lean_object* l_Lean_Elab_Tactic_evalDecideCore_diagnose___lambda__4___clo uint8_t l_Lean_KVMap_getBool(lean_object*, lean_object*, uint8_t); 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_evalNativeDecide(lean_object*); +uint8_t l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_withCollectingNewGoalsFrom(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_type(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalApplyLikeTactic___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*); @@ -18130,7 +18130,7 @@ if (x_5 == 0) lean_object* x_6; lean_object* x_7; uint8_t x_8; x_6 = lean_ctor_get(x_2, 0); x_7 = lean_ctor_get(x_2, 1); -x_8 = l_Array_contains___at_Lean_findField_x3f___spec__1(x_1, x_6); +x_8 = l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(x_1, x_6); if (x_8 == 0) { lean_free_object(x_2); @@ -18158,7 +18158,7 @@ x_12 = lean_ctor_get(x_2, 1); lean_inc(x_12); lean_inc(x_11); lean_dec(x_2); -x_13 = l_Array_contains___at_Lean_findField_x3f___spec__1(x_1, x_11); +x_13 = l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(x_1, x_11); if (x_13 == 0) { lean_dec(x_11); diff --git a/stage0/stdlib/Lean/Elab/Tactic/Ext.c b/stage0/stdlib/Lean/Elab/Tactic/Ext.c index 30b95bca24a0..56055725d6a5 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/Ext.c +++ b/stage0/stdlib/Lean/Elab/Tactic/Ext.c @@ -15,230 +15,217 @@ extern "C" { #endif LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_withExtHyps___spec__2(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_createNodes___rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheorem_declRange__1___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_mkExtType___closed__6; lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_mkExtType___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_evalPrio(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Elab_Tactic_Ext_evalExt___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_Ext_withExtN___spec__4___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__3___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkEqHEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l___private_Lean_Meta_DiscrTreeTypes_0__Lean_Meta_DiscrTree_beqKey____x40_Lean_Meta_DiscrTreeTypes___hyg_101_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_Ext_tryIntros___spec__1___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_evalExt___lambda__2___closed__1; lean_object* l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__1___closed__2; lean_object* l_Lean_Name_reprPrec(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__3; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalExt__1(lean_object*); -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__29; LEAN_EXPORT lean_object* l_Lean_getConstInfoInduct___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__17; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__13; +static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__4; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__12; uint8_t l_Lean_PersistentHashMap_contains___at_Lean_NameSSet_contains___spec__2(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__19; lean_object* l_Lean_MapDeclarationExtension_insert___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_applyExtTheoremAt___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5; lean_object* l_Lean_getConstInfo___at_Lean_Meta_mkConstWithFreshMVarLevels___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__30; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__27; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__1___lambda__1___closed__6; lean_object* lean_mk_empty_array_with_capacity(lean_object*); lean_object* l_Lean_mkAppN(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_applyExtTheoremAt___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__9___closed__1; size_t lean_usize_shift_right(size_t, size_t); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__32; -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__19; lean_object* l_Lean_addBuiltinDocString(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__5___closed__3; static lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___lambda__2___closed__1; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__14; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheorem__1___closed__4; lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__15; +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__7(lean_object*, lean_object*, lean_object*, lean_object*, 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*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__5___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_evalApplyExtTheorem___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheorem_docString__1(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__8___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__35; -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insert___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__5(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3163____boxed(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*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__4___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_tryIntros___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_declRangeExt; lean_object* l_Lean_Elab_Tactic_RCases_rintro(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__28; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_tryIntros___rarg___lambda__4(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__1; +static lean_object* l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__1___closed__4; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__7; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__18; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__59; -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_ConstantInfo_type(lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__25; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_tryIntros___rarg___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__7___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_Ext_withExtHyps___spec__1___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__7(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_applyExtTheoremAt___lambda__3___closed__1; extern lean_object* l_Lean_maxRecDepthErrorMessage; -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__7; -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__27; uint8_t lean_usize_dec_le(size_t, size_t); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__2; static lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___closed__2; -LEAN_EXPORT uint64_t l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3359_(lean_object*); lean_object* l_Lean_ConstantInfo_levelParams(lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__55; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_evalApplyExtTheorem___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7___closed__2; -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__21; -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191_(lean_object*, lean_object*); lean_object* l_Lean_indentD(lean_object*); uint8_t l_Lean_Exception_isInterrupt(lean_object*); static lean_object* l_Lean_Linter_logLint___at_Lean_Elab_Tactic_Ext_evalExt___spec__3___closed__5; uint64_t lean_uint64_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__3(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint64_t lean_uint64_mix_hash(uint64_t, uint64_t); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExt1___at_Lean_Elab_Tactic_Ext_withExtN___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__19; lean_object* l_Lean_mkIff(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__22; lean_object* l_Lean_Meta_isExprDefEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__7(size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_FileMap_toPosition(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__17; size_t lean_uint64_to_usize(uint64_t); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_Ext_ExtTheorems_erase___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__6; -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__23; lean_object* lean_array_fswap(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_logAt___at_Lean_Elab_Tactic_closeUsingOrAdmit___spec__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isAppOfArity(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_Ext_extCore___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExt1___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__7; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__44; static lean_object* l_Lean_Elab_Tactic_Ext_evalExt___lambda__2___closed__4; static lean_object* l_Lean_Elab_Tactic_Ext_applyExtTheoremAt___lambda__2___closed__3; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__7___closed__2; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3253____spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheorem_declRange__1___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_elabTermEnsuringType(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Elab_Tactic_tacticElabAttribute; -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__11; lean_object* l_Array_findIdx_x3f_loop___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__1___lambda__1___closed__4; lean_object* l_Lean_MessageData_ofList(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_Ext_extCore___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__13; lean_object* l_Array_toSubarray___rarg(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__16; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_instBEqExtTheorem___closed__1; static lean_object* l_Lean_Elab_Tactic_Ext_evalExt___lambda__2___closed__5; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___closed__4; size_t lean_usize_mul(size_t, size_t); lean_object* l_Lean_PersistentHashMap_insert___at_Lean_NameSSet_insert___spec__2(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_DiscrTree_instInhabited(lean_object*); -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__4; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__31; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_mk_array(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__21; uint8_t lean_usize_dec_eq(size_t, size_t); static lean_object* l_Lean_Elab_Tactic_Ext_extExt_config___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__12(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_Ext_getExtTheorems___spec__3(lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_DiscrTree_Trie_foldValuesM___at_Lean_Elab_Tactic_Ext_ExtTheorems_erase___spec__1___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getArgs(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtN___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Ext_applyExtTheoremAt___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6(lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_replaceRef(lean_object*, lean_object*); lean_object* l_Lean_MVarId_getType_x27(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___lambda__4(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalExt_declRange__1(lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_mkExtType___closed__3; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__5; lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_eraseCore(lean_object*, lean_object*); -lean_object* l_Lean_Syntax_getPos_x3f(lean_object*, uint8_t); +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__23; lean_object* lean_array_fget(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtN___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_Ext_ExtTheorems_erase___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_forallTelescope___at_Lean_Meta_mapForallTelescope_x27___spec__1___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__1___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Syntax_getTailPos_x3f(lean_object*, uint8_t); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__21; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__8; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__5; +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___lambda__3(size_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_getMainGoal(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_Ext_tryIntros___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__12; -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__22; +LEAN_EXPORT uint64_t l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3253_(lean_object*); +static size_t l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__3___closed__2; lean_object* l_Lean_Expr_fvarId_x21(lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__4; -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_tryIntros___at_Lean_Elab_Tactic_Ext_extCore___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__1; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__19; +lean_object* lean_environment_find(lean_object*, lean_object*); lean_object* l_ReaderT_read___at_Lean_Macro_instMonadRefMacroM___spec__1(lean_object*, lean_object*); -static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__2; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__29; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__38; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_instInhabitedExtTheorem; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__9___closed__2; +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__21; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheorem_docString__1___closed__1; lean_object* l_Lean_addBuiltinDeclarationRanges(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheorem__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_forallTelescopeReducing___at_Lean_Meta_getParamNames___spec__2___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__3(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__6(lean_object*, size_t, size_t, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__2___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__3(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PersistentHashMap_foldlMAux___at_Lean_mkModuleData___spec__3___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Elab_Tactic_Ext_mkExtType___spec__1(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__8(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__20; +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_node5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Nat_nextPowerOfTwo_go(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__11; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__1; lean_object* l_Lean_stringToMessageData(lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_Tactic_Ext_evalExt___spec__2(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__36; static lean_object* l_Lean_Elab_Tactic_Ext_applyExtTheoremAt___lambda__2___closed__1; -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__1; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__16; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_MapDeclarationExtension_contains___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__2; lean_object* l_Lean_RBNode_findCore___at_Lean_Meta_mkGeneralizationForbiddenSet_visit___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtN___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__2(lean_object*, lean_object*); uint8_t lean_string_dec_eq(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheorem_declRange__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_throwError___at_Lean_Meta_setInlineAttribute___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7___closed__1; lean_object* l_Lean_Exception_toMessageData(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____boxed(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__10; +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___closed__4; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExt1___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType___lambda__3___closed__7; lean_object* l_Lean_Expr_appArg_x21(lean_object*); @@ -248,125 +235,129 @@ LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_Ext_tryIntros__ static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalExt_declRange__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_applyExtTheoremAt___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExt1___at_Lean_Elab_Tactic_Ext_extCore___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__21; lean_object* l_Lean_getStructureFields(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___lambda__4___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__16; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__14; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__12; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__2(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__7; +static lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__6___closed__1; uint8_t l_Lean_Expr_hasMVar(lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase(lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__3; static lean_object* l_Lean_Elab_Tactic_Ext_applyExtTheoremAt___lambda__1___closed__1; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__4; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__1(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__7; static lean_object* l_Lean_Linter_logLint___at_Lean_Elab_Tactic_Ext_evalExt___spec__3___closed__1; +LEAN_EXPORT uint8_t l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3163_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExt1___at_Lean_Elab_Tactic_Ext_withExtN___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_extCore(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___lambda__4___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__2; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__5; +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__5; +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__1___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365_(lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__2; LEAN_EXPORT uint8_t l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___rarg___lambda__2(lean_object*, uint8_t, lean_object*); lean_object* l_Lean_Elab_Tactic_RCases_expandRIntroPats(lean_object*, lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType___lambda__2___closed__4; -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___rarg(lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_mkExtType___closed__5; lean_object* l_Lean_FVarId_getBinderInfo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__34; -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__10; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__1; +static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__5; static lean_object* l_Lean_Linter_logLint___at_Lean_Elab_Tactic_Ext_evalExt___spec__3___closed__3; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_Ext_evalExt___spec__1(size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766_(lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__3___closed__1; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__8; -LEAN_EXPORT lean_object* l_Std_Format_joinSep___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____spec__2(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_repr___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_getExtTheorems(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_logLint___at_Lean_Elab_Tactic_Ext_evalExt___spec__3___closed__6; -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3269____boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__9; lean_object* l_Array_reverse___rarg(lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__17; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__14; -static lean_object* l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__1; -lean_object* l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_throwError___at_Lean_Expr_abstractRangeM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__50; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__9(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheorem_declRange__1(lean_object*); -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__8; +static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__3; lean_object* lean_st_ref_take(lean_object*, lean_object*); lean_object* l_Lean_Expr_getRevArg_x21(lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__1___closed__2; lean_object* l_liftExcept___at_Lean_Elab_liftMacroM___spec__1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__2; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__4; static lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType___lambda__4___closed__1; static lean_object* l_Lean_Elab_Tactic_Ext_mkExtType___closed__1; lean_object* l_Lean_Elab_expandMacroImpl_x3f(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__2(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_instInhabitedExtTheorems___closed__1; -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__15; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__3; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__15; uint8_t lean_expr_eqv(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__7; lean_object* l_Lean_ResolveName_resolveNamespace(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__28; lean_object* l_Lean_registerSimpleScopedEnvExtension___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__25; +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6(lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__9___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_tryIntros___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__31; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__1; lean_object* l_Lean_SourceInfo_fromRef(lean_object*, uint8_t); -LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_ReaderT_bind___at_Lean_Macro_instMonadRefMacroM___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_to_int(lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__1; lean_object* l_Lean_MessageData_ofSyntax(lean_object*); lean_object* l_Lean_Syntax_node6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__24; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__15; lean_object* lean_nat_div(lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__26; static lean_object* l_Lean_Linter_logLint___at_Lean_Elab_Tactic_Ext_evalExt___spec__3___closed__4; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__5; lean_object* l_Lean_getConstInfo___at_Lean_Elab_Term_mkConst___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtN___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallMetaTelescopeReducingAux(lean_object*, uint8_t, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__2___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_instHashableExtTheorem___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__1___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Format_joinSep___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____spec__2(lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_withoutErrToSorryImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___closed__5; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_withExtHyps___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__4(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__5; static lean_object* l_Lean_getConstInfoInduct___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__1___closed__2; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__7; LEAN_EXPORT uint8_t l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___rarg___lambda__3(lean_object*, uint8_t, lean_object*, lean_object*); +static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__3; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__4(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_SavedState_restore(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Command_getRef(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Elab_Tactic_Ext_mkExtType___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__18; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__18; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_tryIntros___rarg___lambda__6___closed__2; static lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType___lambda__3___closed__8; -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____lambda__1(lean_object*, lean_object*); lean_object* l_Lean_Meta_withNewMCtxDepth___at_Lean_Meta_matchesInstance___spec__1___rarg(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9___closed__1; lean_object* l_Lean_MessageData_ofFormat(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkCIdentFrom(lean_object*, lean_object*, uint8_t); lean_object* l_Lean_Elab_getBetterRef(lean_object*, lean_object*); uint8_t l_Lean_Expr_isMVar(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalExt_declRange__1___closed__2; lean_object* l_Lean_MVarId_withContext___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_synthPendingImp___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_tryIntros___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_binInsertM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__11(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_insertVal_loop___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__10(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__33; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__15; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__11; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_Ext_withExtN___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -374,100 +365,108 @@ lean_object* l_Lean_Expr_forallE___override(lean_object*, lean_object*, lean_obj lean_object* l_outOfBounds___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps(lean_object*); lean_object* l_Lean_Elab_Tactic_withMainContext___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__18; static lean_object* l_Lean_Elab_Tactic_Ext_applyExtTheoremAt___lambda__2___closed__2; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__13; +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__30; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__63; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__60; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_applyExtTheoremAt(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Command_liftTermElabM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___lambda__5(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__7; lean_object* lean_st_ref_get(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__3___closed__2; lean_object* l_Lean_throwError___at_Lean_registerTagAttribute___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_tryIntros___rarg___lambda__6___closed__4; lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_liftCommandElabM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_liftCommandElabM___rarg(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkAndN(lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_applyExtTheoremAt___lambda__3___closed__2; lean_object* l_Lean_Syntax_getOptional_x3f(lean_object*); lean_object* lean_st_mk_ref(lean_object*, lean_object*); -static lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__6___closed__1; -static lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___rarg___closed__2; +static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5; lean_object* lean_array_to_list(lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__6; lean_object* l_ReaderT_instApplicativeOfMonad___rarg(lean_object*); lean_object* l_Lean_Meta_mkEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__13; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__3___closed__3; +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__2; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Ext_applyExtTheoremAt___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__1; static lean_object* l_Lean_Elab_Tactic_Ext_getExtTheorems___closed__1; -static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__5; -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3359____boxed(lean_object*); lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); lean_object* l_Lean_Syntax_node3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__4; -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__9; lean_object* l_Lean_ScopedEnvExtension_modifyState___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__24; -static lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___rarg___closed__1; static lean_object* l_Lean_Elab_Tactic_Ext_mkExtType___closed__4; static lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_evalExt___closed__1; -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__12; +static lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__5___rarg___closed__2; +static lean_object* l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__1___closed__3; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__57; +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Meta_DiscrTree_Key_lt(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__3(lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_tryIntros___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__15; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_mkExtType___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__16; static lean_object* l_Lean_Elab_Tactic_Ext_instReprExtTheorem___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__2(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__5___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__5(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__2; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_applyExtTheoremAt___spec__1___closed__1; -static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__1; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__3; lean_object* l_Lean_Elab_Command_getCurrMacroScope(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__13___closed__1; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__20; +LEAN_EXPORT uint64_t l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3253____spec__1(lean_object*, size_t, size_t, uint64_t); +LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__9(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_applyExtTheoremAt___closed__2; static lean_object* l_Lean_Elab_Tactic_Ext_mkExtType___closed__8; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085_(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__13; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__10; static lean_object* l_Lean_Elab_Tactic_Ext_evalExt___lambda__2___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__13(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_binInsertM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addMacroScope(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__1; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__5; +LEAN_EXPORT lean_object* l_List_foldl___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____spec__3(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ScopedEnvExtension_add___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__6(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__4___closed__2; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__4; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insert___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__5(lean_object*, lean_object*, lean_object*); uint8_t lean_name_eq(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__26; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__54; -LEAN_EXPORT lean_object* l_repr___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____spec__1(lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__9; static lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___lambda__3___closed__1; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__1; static lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___rarg___closed__2; -static size_t l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_tryIntros___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__4; lean_object* l_Lean_Syntax_node2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_instInhabitedExtTheorems; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType___lambda__1___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__2; +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__16; +LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__4; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___closed__1; -LEAN_EXPORT uint8_t l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3269_(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__1; static lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType___lambda__3___closed__6; +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__3; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__14; lean_object* l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); @@ -475,7 +474,6 @@ lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_evalExt(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__37; uint8_t l_Lean_Syntax_matchesNull(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__5; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__17; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__5; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_Ext_tryIntros___spec__1___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); @@ -483,79 +481,79 @@ LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_Ext_withExtN___ LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_Tactic_Ext_evalExt___spec__2___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_saveState___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtN___at_Lean_Elab_Tactic_Ext_extCore___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType___lambda__3___closed__4; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__23; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__5___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_mkExtType(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_extExt_config; +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__25; lean_object* l_Lean_Expr_appFn_x21(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_mkExtType___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Command_getScope___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_instHashableExtTheorem; lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_withSynthesizeImp___rarg(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_CollectFVars_main(lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_applyExtTheoremAt___spec__1___lambda__1___closed__1; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__46; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____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_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_Ext_withExt1___spec__1(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__8___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutErrToSorry___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__1___closed__1; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__4; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__52; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__30; LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_foldlM___at_Lean_Elab_Tactic_Ext_ExtTheorems_erase___spec__6(lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExt1___at_Lean_Elab_Tactic_Ext_withExtN___spec__3(lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__6; -static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__3; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__53; lean_object* l_Lean_Meta_DiscrTree_mkPath(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_usize_to_nat(size_t); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheorem__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExt1___at_Lean_Elab_Tactic_Ext_withExtN___spec__3___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkConstWithLevelParams___at_Lean_Meta_mkSimpCongrTheorem___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_Tactic_Ext_mkExtIffType___lambda__1(lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofConstName(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__8___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); -lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Environment_contains(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__17; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__47; -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__6; +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__28; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__8; -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3(lean_object*, size_t, lean_object*); lean_object* l_Lean_MessageData_ofExpr(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__1___lambda__1___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_insertionSort_swapLoop___at_Lean_Elab_Tactic_Ext_getExtTheorems___spec__2(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtN___at_Lean_Elab_Tactic_Ext_extCore___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__8___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_getConstInfo___at_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___spec__1___closed__2; lean_object* l_instMonadControlTOfPure___rarg(lean_object*); +static lean_object* l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__13___closed__1; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__5; -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__2; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__11; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__10; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__33; static lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType___lambda__2___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__2___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_throwError___at_Lean_Meta_mkSimpCongrTheorem___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_foldlM___at_Lean_Elab_Tactic_Ext_ExtTheorems_erase___spec__6___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_tryIntros(lean_object*); lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_SynthInstance_removeUnusedArguments_x3f___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___lambda__1(lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_applyExtTheoremAt___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__4; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660_(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_Ext_getExtTheorems___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_node4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_getConstInfoInduct___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__1___closed__1; -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__17; static lean_object* l_Lean_Elab_Tactic_Ext_evalExt___lambda__2___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutErrToSorry___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ScopedEnvExtension_add___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_extCore___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__13(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_applyExtTheoremAt___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__43; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalExt__1___closed__2; -LEAN_EXPORT uint8_t l_Array_isEqvAux___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3269____spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_evalExt___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_FileMap_leanPosToLspPos(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__34; @@ -564,66 +562,69 @@ static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheorem__1__ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_tryIntros___rarg___lambda__2(lean_object*, lean_object*); static lean_object* l_Lean_getConstInfoInduct___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__1___closed__4; static lean_object* l_Lean_Elab_Tactic_Ext_applyExtTheoremAt___closed__3; +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__3(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalExt_declRange__1___closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__5(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__26; LEAN_EXPORT uint8_t l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_Ext_ExtTheorems_erase___spec__2(lean_object*, lean_object*, size_t, size_t, uint8_t); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__1___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__12; +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_evalApplyExtTheorem___rarg___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_Ext_applyExtTheoremAt___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_getExtTheorems___closed__2; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__7; lean_object* l_Lean_throwError___rarg(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__2; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__10; extern lean_object* l_Lean_Meta_DiscrTree_instInhabitedKey; static lean_object* l_Lean_Elab_Tactic_Ext_tryIntros___rarg___lambda__6___closed__1; static lean_object* l_Lean_Linter_logLint___at_Lean_Elab_Tactic_Ext_evalExt___spec__3___closed__2; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__24; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___closed__2; uint8_t l_Lean_Name_isAtomic(lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__16; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__4___closed__1; static lean_object* l_Lean_Elab_Tactic_Ext_mkExtType___closed__2; lean_object* lean_string_length(lean_object*); -static lean_object* l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__3; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___closed__6; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__19; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__9; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheorem__1___closed__6; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_TSyntax_getNat(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_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_instReprExtTheorem; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_Ext_withExtN___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__21; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__12___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_instInhabitedExtTheorem___closed__1; uint8_t lean_nat_dec_lt(lean_object*, lean_object*); -static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__4; +LEAN_EXPORT lean_object* l_Array_isEqvAux___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3163____spec__1___boxed(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_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_Ext_applyExtTheoremAt___spec__3(lean_object*, lean_object*, size_t, size_t, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__20; LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Elab_Tactic_Ext_evalExt___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalExt_declRange__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_Ext_tryIntros___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__58; -static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__3; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_Ext_evalExt___spec__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___rarg___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_id___rarg___boxed(lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__8; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtN___at_Lean_Elab_Tactic_Ext_extCore___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_binInsertM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_binInsertM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__1___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType___lambda__3___closed__1; +LEAN_EXPORT lean_object* l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__1___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_indentExpr(lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__3; lean_object* l_List_forM___at_Lean_Elab_Command_elabCommand___spec__8(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PersistentHashMap_mkEmptyEntries(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -631,11 +632,8 @@ lean_object* l___private_Lean_Meta_DiscrTreeTypes_0__Lean_Meta_DiscrTree_reprKey LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___lambda__2(lean_object*, size_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_node7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__3; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__2; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__6; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__6(lean_object*, size_t, size_t, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__39; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__2; lean_object* l_Lean_Syntax_node1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_evalApplyExtTheorem___boxed(lean_object*); lean_object* l_Lean_TagDeclarationExtension_tag(lean_object*, lean_object*, lean_object*); @@ -643,67 +641,72 @@ static lean_object* l_Lean_Elab_Tactic_Ext_applyExtTheoremAt___lambda__1___close LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_Ext_withExtN___spec__4(lean_object*); lean_object* l_Lean_Meta_mkForallFVars(lean_object*, lean_object*, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__5___closed__2; -LEAN_EXPORT lean_object* l_Lean_ScopedEnvExtension_add___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__6(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__1___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__13(lean_object*, lean_object*, lean_object*, lean_object*); uint64_t l_Lean_Name_hash___override(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalExt__1___closed__1; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__8; uint8_t l_Lean_Syntax_isNone(lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__4___closed__2; lean_object* lean_panic_fn(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_evalApplyExtTheorem(lean_object*); +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__9; +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_insertionSort_traverse___at_Lean_Elab_Tactic_Ext_getExtTheorems___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___lambda__4___boxed__const__1; -static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____lambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_ResolveName_resolveGlobalName(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__24; -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__8(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__13; lean_object* l_Lean_ScopedEnvExtension_getState___rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__8(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__1; lean_object* l_Array_insertAt_x21___rarg(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_withLCtx___at___private_Lean_Meta_Basic_0__Lean_Meta_mkLevelErrorMessageCore___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_isStructure(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_applyExtTheoremAt___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_applyExtTheoremAt___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Array_isEqvAux___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3163____spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Syntax_getRange_x3f(lean_object*, uint8_t); lean_object* l_Lean_ScopedEnvExtension_addCore___rarg(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_evalExt___lambda__2___closed__6; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType___lambda__3___closed__5; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getConstInfoInduct___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PersistentHashMap_mkCollisionNode___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__11; static lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType___lambda__2___closed__3; LEAN_EXPORT uint8_t l_Lean_Meta_DiscrTree_Trie_foldValuesM___at_Lean_Elab_Tactic_Ext_ExtTheorems_erase___spec__1(lean_object*, uint8_t, lean_object*); -static lean_object* l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__2; static lean_object* l_Lean_Elab_Tactic_Ext_tryIntros___rarg___lambda__6___closed__3; -static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__6; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheorem__1___closed__3; extern lean_object* l_Lean_Elab_Tactic_RCases_linter_unusedRCasesPattern; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__49; lean_object* l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); lean_object* l_Array_ofSubarray___rarg(lean_object*); -static size_t l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3___closed__1; extern lean_object* l_Lean_Core_instMonadCoreM; lean_object* l_Lean_MVarId_apply(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ScopedEnvExtension_add___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__5___rarg___closed__1; static lean_object* l_Lean_Elab_Tactic_Ext_applyExtTheoremAt___closed__1; extern lean_object* l_Lean_protectedExt; extern lean_object* l_Lean_instInhabitedDeclarationRanges; lean_object* l_Lean_registerBuiltinAttribute(lean_object*, lean_object*); lean_object* l_Array_back___rarg(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_Ext_ExtTheorems_erase___spec__4(lean_object*, lean_object*, size_t, size_t, uint8_t); +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__1(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_getConstInfo___at_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___spec__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_reverse___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_evalExt___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__14; +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__10; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtN___at_Lean_Elab_Tactic_Ext_extCore___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__32; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__23; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_extCore___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -714,44 +717,45 @@ lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalRepeat static lean_object* l_Lean_getConstInfoInduct___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__1___closed__3; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_Ext_withExtN___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_applyExtTheoremAt___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__2; lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_SynthInstance_removeUnusedArguments_x3f___spec__2___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__45; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExt1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__5; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_extExtension; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExt1___rarg___lambda__2(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); -static lean_object* l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_extCore___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_tryIntros___rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExt1(lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_evalApplyExtTheorem___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__3___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_evalExt___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__27; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__6; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__7(size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_evalExt___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__2___boxed(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalExt__1___closed__3; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__19; lean_object* lean_array_uget(lean_object*, size_t); -LEAN_EXPORT uint64_t l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3359____spec__1(lean_object*, size_t, size_t, uint64_t); size_t lean_array_size(lean_object*); +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__14; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__8(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__3; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__1___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_Ext_withExtHyps___spec__1(size_t, size_t, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_tryIntros___rarg___lambda__4___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___closed__1; lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__12___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__29; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__6; size_t lean_usize_shift_left(size_t, size_t); -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__1___lambda__1___closed__2; lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -759,74 +763,79 @@ static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalExt_declRange__1___c static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__62; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__1___lambda__1___closed__3; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__12; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__3___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__4; +static size_t l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__3___closed__1; lean_object* lean_string_append(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10(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_Lean_Elab_Tactic_Ext_withExt1___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__2; LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_Ext_withExt1___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheorem_declRange__1___closed__7; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__8; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__18; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_Ext_ExtTheorems_erase___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_evalExt___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3359____spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__41; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__40; lean_object* lean_array_get_size(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheorem__1___closed__5; -LEAN_EXPORT lean_object* l_List_foldl___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____spec__3(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_mkExtType___closed__7; +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__5___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_instBEqExtTheorem; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__48; -LEAN_EXPORT lean_object* l___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType___lambda__3___closed__3; lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_arrowDomainsN___spec__1(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_Ext_ExtTheorems_erase___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtN___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__22; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtN(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExt1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); extern lean_object* l_Lean_Elab_unsupportedSyntaxExceptionId; uint8_t lean_usize_dec_lt(size_t, size_t); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__2; LEAN_EXPORT uint8_t l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_Ext_ExtTheorems_erase___spec__5(lean_object*, lean_object*, size_t, size_t, uint8_t); -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__7; +lean_object* l_Lean_throwError___at_Lean_withSetOptionIn___spec__7(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkProjection(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__1___lambda__1___closed__1; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__5; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__51; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MVarId_intros(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PersistentHashMap_erase___at_Lean_Meta_addInstanceEntry___spec__18(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertVal_loop___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__10(lean_object*, lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__1___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PersistentHashMap_getCollisionNodeSize___rarg(lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__4; uint8_t l_Lean_Exception_isRuntime(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__1___lambda__1___closed__7; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3253____boxed(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheorem_declRange__1___closed__6; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__4; lean_object* l_Lean_Meta_DiscrTree_getMatch___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__29; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__9; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__30; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheorem_declRange__1___closed__2; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__61; -LEAN_EXPORT lean_object* l___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_extCore___closed__1; uint8_t l_Lean_Expr_isForall(lean_object*); lean_object* l_Lean_Meta_mkConstWithFreshMVarLevels(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_getStructureFieldsFlattened(lean_object*, lean_object*, uint8_t); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__5___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_tryIntros___rarg___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_String_toSubstring_x27(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_applyExtTheoremAt___spec__1___lambda__1___closed__2; -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__25; -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__13(lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__18; static lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType___lambda__3___closed__2; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__20; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtN___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExt1___at_Lean_Elab_Tactic_Ext_withExtN___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MVarId_withContext___at_Lean_Elab_Tactic_run___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -834,36 +843,34 @@ lean_object* l_Lean_MessageData_ofName(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExt1___at_Lean_Elab_Tactic_Ext_withExtN___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_get(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_replaceMainGoal(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__6; lean_object* l___private_Init_Data_Repr_0__Nat_reprFast(lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__7; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____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*); uint64_t l_Lean_Meta_DiscrTree_Key_hash(lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__6; -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__26; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__5; +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__8; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__22; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_Ext_tryIntros___spec__1(lean_object*); +static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__1; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__20; +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__4; lean_object* l_Lean_Meta_isProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addDecl(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_ReaderT_instMonad___rarg(lean_object*); extern lean_object* l_Lean_PersistentHashMap_empty___at_Lean_Meta_Match_instInhabitedMatchEqnsExtState___spec__1; +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__27; size_t lean_usize_land(size_t, size_t); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__7; -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__11; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_applyExtTheoremAt___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_withNewBinderInfos___at_Lean_Meta_withInstImplicitAsImplict___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_isEqvAux___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3269____spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__28; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__1; lean_object* l_ReaderT_pure___at_Lean_Elab_liftMacroM___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalExt_declRange__1___closed__7; static lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__12(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_Ext_ExtTheorems_erase___spec__3(lean_object*, lean_object*, size_t, size_t, uint8_t); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Array_isEmpty___rarg(lean_object*); +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__20; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___closed__3; lean_object* l_Lean_Elab_Term_withDeclName___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_Ext_withExtHyps___spec__1(size_t x_1, size_t x_2, lean_object* x_3) { @@ -3565,242 +3572,151 @@ return x_29; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_9; uint8_t x_10; lean_object* x_11; lean_object* x_12; -x_9 = lean_ctor_get(x_6, 1); -lean_inc(x_9); -lean_dec(x_6); -x_10 = 0; -x_11 = l_Lean_Syntax_getPos_x3f(x_1, x_10); -x_12 = l_Lean_Syntax_getTailPos_x3f(x_1, x_10); -if (lean_obj_tag(x_11) == 0) +uint8_t x_9; lean_object* x_10; +x_9 = 0; +x_10 = l_Lean_Syntax_getRange_x3f(x_1, x_9); +if (lean_obj_tag(x_10) == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_unsigned_to_nat(0u); -lean_inc(x_9); -x_14 = l_Lean_FileMap_toPosition(x_9, x_13); -lean_inc(x_14); -x_15 = l_Lean_FileMap_leanPosToLspPos(x_9, x_14); -if (lean_obj_tag(x_12) == 0) +lean_object* x_11; lean_object* x_12; +lean_dec(x_6); +x_11 = lean_box(0); +x_12 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_11); +lean_ctor_set(x_12, 1, x_8); +return x_12; +} +else { -uint8_t x_16; -lean_dec(x_9); -x_16 = !lean_is_exclusive(x_15); -if (x_16 == 0) +uint8_t x_13; +x_13 = !lean_is_exclusive(x_10); +if (x_13 == 0) { -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_15, 1); -x_18 = lean_ctor_get(x_15, 0); +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_14 = lean_ctor_get(x_10, 0); +x_15 = lean_ctor_get(x_6, 1); +lean_inc(x_15); +lean_dec(x_6); +x_16 = lean_ctor_get(x_14, 0); +lean_inc(x_16); +lean_inc(x_15); +x_17 = l_Lean_FileMap_toPosition(x_15, x_16); +lean_dec(x_16); +x_18 = lean_ctor_get(x_14, 1); +lean_inc(x_18); +lean_dec(x_14); +lean_inc(x_15); +x_19 = l_Lean_FileMap_toPosition(x_15, x_18); lean_dec(x_18); lean_inc(x_17); -lean_inc(x_14); -x_19 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_19, 0, x_14); -lean_ctor_set(x_19, 1, x_17); -lean_ctor_set(x_19, 2, x_14); -lean_ctor_set(x_19, 3, x_17); -lean_ctor_set(x_15, 1, x_8); -lean_ctor_set(x_15, 0, x_19); -return x_15; -} -else +x_20 = l_Lean_FileMap_leanPosToLspPos(x_15, x_17); +x_21 = !lean_is_exclusive(x_20); +if (x_21 == 0) { -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_15, 1); -lean_inc(x_20); +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_22 = lean_ctor_get(x_20, 1); +x_23 = lean_ctor_get(x_20, 0); +lean_dec(x_23); +lean_inc(x_19); +x_24 = l_Lean_FileMap_leanPosToLspPos(x_15, x_19); lean_dec(x_15); -lean_inc(x_20); -lean_inc(x_14); -x_21 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_21, 0, x_14); -lean_ctor_set(x_21, 1, x_20); -lean_ctor_set(x_21, 2, x_14); -lean_ctor_set(x_21, 3, x_20); -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_21); -lean_ctor_set(x_22, 1, x_8); -return x_22; -} +x_25 = lean_ctor_get(x_24, 1); +lean_inc(x_25); +lean_dec(x_24); +x_26 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_26, 0, x_17); +lean_ctor_set(x_26, 1, x_22); +lean_ctor_set(x_26, 2, x_19); +lean_ctor_set(x_26, 3, x_25); +lean_ctor_set(x_10, 0, x_26); +lean_ctor_set(x_20, 1, x_8); +lean_ctor_set(x_20, 0, x_10); +return x_20; } else { -uint8_t x_23; -x_23 = !lean_is_exclusive(x_15); -if (x_23 == 0) -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_24 = lean_ctor_get(x_15, 1); -x_25 = lean_ctor_get(x_15, 0); -lean_dec(x_25); -x_26 = lean_ctor_get(x_12, 0); -lean_inc(x_26); -lean_dec(x_12); -lean_inc(x_9); -x_27 = l_Lean_FileMap_toPosition(x_9, x_26); -lean_dec(x_26); +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_27 = lean_ctor_get(x_20, 1); lean_inc(x_27); -x_28 = l_Lean_FileMap_leanPosToLspPos(x_9, x_27); -lean_dec(x_9); +lean_dec(x_20); +lean_inc(x_19); +x_28 = l_Lean_FileMap_leanPosToLspPos(x_15, x_19); +lean_dec(x_15); x_29 = lean_ctor_get(x_28, 1); lean_inc(x_29); lean_dec(x_28); x_30 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_30, 0, x_14); -lean_ctor_set(x_30, 1, x_24); -lean_ctor_set(x_30, 2, x_27); +lean_ctor_set(x_30, 0, x_17); +lean_ctor_set(x_30, 1, x_27); +lean_ctor_set(x_30, 2, x_19); lean_ctor_set(x_30, 3, x_29); -lean_ctor_set(x_15, 1, x_8); -lean_ctor_set(x_15, 0, x_30); -return x_15; +lean_ctor_set(x_10, 0, x_30); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_10); +lean_ctor_set(x_31, 1, x_8); +return x_31; +} } else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_31 = lean_ctor_get(x_15, 1); -lean_inc(x_31); -lean_dec(x_15); -x_32 = lean_ctor_get(x_12, 0); +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_32 = lean_ctor_get(x_10, 0); lean_inc(x_32); -lean_dec(x_12); -lean_inc(x_9); -x_33 = l_Lean_FileMap_toPosition(x_9, x_32); +lean_dec(x_10); +x_33 = lean_ctor_get(x_6, 1); +lean_inc(x_33); +lean_dec(x_6); +x_34 = lean_ctor_get(x_32, 0); +lean_inc(x_34); +lean_inc(x_33); +x_35 = l_Lean_FileMap_toPosition(x_33, x_34); +lean_dec(x_34); +x_36 = lean_ctor_get(x_32, 1); +lean_inc(x_36); lean_dec(x_32); lean_inc(x_33); -x_34 = l_Lean_FileMap_leanPosToLspPos(x_9, x_33); -lean_dec(x_9); -x_35 = lean_ctor_get(x_34, 1); +x_37 = l_Lean_FileMap_toPosition(x_33, x_36); +lean_dec(x_36); lean_inc(x_35); -lean_dec(x_34); -x_36 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_36, 0, x_14); -lean_ctor_set(x_36, 1, x_31); -lean_ctor_set(x_36, 2, x_33); -lean_ctor_set(x_36, 3, x_35); -x_37 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_37, 0, x_36); -lean_ctor_set(x_37, 1, x_8); -return x_37; -} -} -} -else -{ -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_11, 0); -lean_inc(x_38); -lean_dec(x_11); -lean_inc(x_9); -x_39 = l_Lean_FileMap_toPosition(x_9, x_38); -lean_dec(x_38); -lean_inc(x_39); -x_40 = l_Lean_FileMap_leanPosToLspPos(x_9, x_39); -if (lean_obj_tag(x_12) == 0) -{ -uint8_t x_41; -lean_dec(x_9); -x_41 = !lean_is_exclusive(x_40); -if (x_41 == 0) -{ -lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_ctor_get(x_40, 1); -x_43 = lean_ctor_get(x_40, 0); -lean_dec(x_43); -lean_inc(x_42); -lean_inc(x_39); -x_44 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_44, 0, x_39); -lean_ctor_set(x_44, 1, x_42); -lean_ctor_set(x_44, 2, x_39); -lean_ctor_set(x_44, 3, x_42); -lean_ctor_set(x_40, 1, x_8); -lean_ctor_set(x_40, 0, x_44); -return x_40; -} -else -{ -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_40, 1); -lean_inc(x_45); -lean_dec(x_40); -lean_inc(x_45); +x_38 = l_Lean_FileMap_leanPosToLspPos(x_33, x_35); +x_39 = lean_ctor_get(x_38, 1); lean_inc(x_39); -x_46 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_46, 0, x_39); -lean_ctor_set(x_46, 1, x_45); -lean_ctor_set(x_46, 2, x_39); -lean_ctor_set(x_46, 3, x_45); -x_47 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_47, 0, x_46); -lean_ctor_set(x_47, 1, x_8); -return x_47; -} -} -else -{ -uint8_t x_48; -x_48 = !lean_is_exclusive(x_40); -if (x_48 == 0) -{ -lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_49 = lean_ctor_get(x_40, 1); -x_50 = lean_ctor_get(x_40, 0); -lean_dec(x_50); -x_51 = lean_ctor_get(x_12, 0); -lean_inc(x_51); -lean_dec(x_12); -lean_inc(x_9); -x_52 = l_Lean_FileMap_toPosition(x_9, x_51); -lean_dec(x_51); -lean_inc(x_52); -x_53 = l_Lean_FileMap_leanPosToLspPos(x_9, x_52); -lean_dec(x_9); -x_54 = lean_ctor_get(x_53, 1); -lean_inc(x_54); -lean_dec(x_53); -x_55 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_55, 0, x_39); -lean_ctor_set(x_55, 1, x_49); -lean_ctor_set(x_55, 2, x_52); -lean_ctor_set(x_55, 3, x_54); -lean_ctor_set(x_40, 1, x_8); -lean_ctor_set(x_40, 0, x_55); -return x_40; +if (lean_is_exclusive(x_38)) { + lean_ctor_release(x_38, 0); + lean_ctor_release(x_38, 1); + x_40 = x_38; +} else { + lean_dec_ref(x_38); + x_40 = lean_box(0); } -else -{ -lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_56 = lean_ctor_get(x_40, 1); -lean_inc(x_56); -lean_dec(x_40); -x_57 = lean_ctor_get(x_12, 0); -lean_inc(x_57); -lean_dec(x_12); -lean_inc(x_9); -x_58 = l_Lean_FileMap_toPosition(x_9, x_57); -lean_dec(x_57); -lean_inc(x_58); -x_59 = l_Lean_FileMap_leanPosToLspPos(x_9, x_58); -lean_dec(x_9); -x_60 = lean_ctor_get(x_59, 1); -lean_inc(x_60); -lean_dec(x_59); -x_61 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_61, 0, x_39); -lean_ctor_set(x_61, 1, x_56); -lean_ctor_set(x_61, 2, x_58); -lean_ctor_set(x_61, 3, x_60); -x_62 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_62, 0, x_61); -lean_ctor_set(x_62, 1, x_8); -return x_62; +lean_inc(x_37); +x_41 = l_Lean_FileMap_leanPosToLspPos(x_33, x_37); +lean_dec(x_33); +x_42 = lean_ctor_get(x_41, 1); +lean_inc(x_42); +lean_dec(x_41); +x_43 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_43, 0, x_35); +lean_ctor_set(x_43, 1, x_39); +lean_ctor_set(x_43, 2, x_37); +lean_ctor_set(x_43, 3, x_42); +x_44 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_44, 0, x_43); +if (lean_is_scalar(x_40)) { + x_45 = lean_alloc_ctor(0, 2, 0); +} else { + x_45 = x_40; } +lean_ctor_set(x_45, 0, x_44); +lean_ctor_set(x_45, 1, x_8); +return x_45; } } } } -static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__1() { +static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__1() { _start: { lean_object* x_1; @@ -3808,7 +3724,7 @@ x_1 = l_Lean_declRangeExt; return x_1; } } -static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__2() { +static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__2() { _start: { lean_object* x_1; lean_object* x_2; @@ -3819,7 +3735,7 @@ lean_ctor_set(x_2, 1, x_1); return x_2; } } -static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__3() { +static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__3() { _start: { lean_object* x_1; lean_object* x_2; @@ -3830,7 +3746,7 @@ lean_ctor_set(x_2, 1, x_1); return x_2; } } -static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__4() { +static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__4() { _start: { lean_object* x_1; lean_object* x_2; @@ -3843,13 +3759,13 @@ lean_ctor_set(x_2, 3, x_1); return x_2; } } -static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5() { +static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__3; +x_1 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__3; x_2 = l_Lean_Elab_Tactic_Ext_mkExtType___closed__2; -x_3 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__4; +x_3 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__4; x_4 = lean_alloc_ctor(0, 7, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -3861,7 +3777,7 @@ lean_ctor_set(x_4, 6, x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { lean_object* x_10; uint8_t x_11; @@ -3876,7 +3792,7 @@ x_14 = lean_ctor_get(x_12, 0); lean_inc(x_14); lean_dec(x_12); x_15 = l_Lean_instInhabitedDeclarationRanges; -x_16 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__1; +x_16 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__1; lean_inc(x_1); x_17 = l_Lean_MapDeclarationExtension_contains___rarg(x_15, x_16, x_14, x_1); lean_dec(x_14); @@ -3898,7 +3814,7 @@ x_22 = lean_ctor_get(x_19, 0); x_23 = lean_ctor_get(x_19, 4); lean_dec(x_23); x_24 = l_Lean_MapDeclarationExtension_insert___rarg(x_16, x_22, x_1, x_2); -x_25 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__2; +x_25 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__2; lean_ctor_set(x_19, 4, x_25); lean_ctor_set(x_19, 0, x_24); x_26 = lean_st_ref_set(x_8, x_19, x_20); @@ -3917,7 +3833,7 @@ if (x_31 == 0) lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; x_32 = lean_ctor_get(x_29, 1); lean_dec(x_32); -x_33 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5; +x_33 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5; lean_ctor_set(x_29, 1, x_33); x_34 = lean_st_ref_set(x_6, x_29, x_30); x_35 = !lean_is_exclusive(x_34); @@ -3955,7 +3871,7 @@ lean_inc(x_43); lean_inc(x_42); lean_inc(x_41); lean_dec(x_29); -x_45 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5; +x_45 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5; x_46 = lean_alloc_ctor(0, 5, 0); lean_ctor_set(x_46, 0, x_41); lean_ctor_set(x_46, 1, x_45); @@ -4001,7 +3917,7 @@ lean_inc(x_53); lean_inc(x_52); lean_dec(x_19); x_58 = l_Lean_MapDeclarationExtension_insert___rarg(x_16, x_52, x_1, x_2); -x_59 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__2; +x_59 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__2; x_60 = lean_alloc_ctor(0, 7, 0); lean_ctor_set(x_60, 0, x_58); lean_ctor_set(x_60, 1, x_53); @@ -4039,7 +3955,7 @@ if (lean_is_exclusive(x_64)) { lean_dec_ref(x_64); x_70 = lean_box(0); } -x_71 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5; +x_71 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5; if (lean_is_scalar(x_70)) { x_72 = lean_alloc_ctor(0, 5, 0); } else { @@ -4094,7 +4010,7 @@ x_81 = lean_ctor_get(x_79, 0); lean_inc(x_81); lean_dec(x_79); x_82 = l_Lean_instInhabitedDeclarationRanges; -x_83 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__1; +x_83 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__1; lean_inc(x_1); x_84 = l_Lean_MapDeclarationExtension_contains___rarg(x_82, x_83, x_81, x_1); lean_dec(x_81); @@ -4133,7 +4049,7 @@ if (lean_is_exclusive(x_86)) { x_94 = lean_box(0); } x_95 = l_Lean_MapDeclarationExtension_insert___rarg(x_83, x_88, x_1, x_2); -x_96 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__2; +x_96 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__2; if (lean_is_scalar(x_94)) { x_97 = lean_alloc_ctor(0, 7, 0); } else { @@ -4175,7 +4091,7 @@ if (lean_is_exclusive(x_101)) { lean_dec_ref(x_101); x_107 = lean_box(0); } -x_108 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5; +x_108 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5; if (lean_is_scalar(x_107)) { x_109 = lean_alloc_ctor(0, 5, 0); } else { @@ -4221,7 +4137,127 @@ return x_116; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutErrToSorry___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; +lean_inc(x_8); +x_11 = l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4(x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +if (lean_obj_tag(x_12) == 0) +{ +uint8_t x_13; +lean_dec(x_8); +lean_dec(x_1); +x_13 = !lean_is_exclusive(x_11); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_11, 0); +lean_dec(x_14); +x_15 = lean_box(0); +lean_ctor_set(x_11, 0, x_15); +return x_11; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_11, 1); +lean_inc(x_16); +lean_dec(x_11); +x_17 = lean_box(0); +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set(x_18, 1, x_16); +return x_18; +} +} +else +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_19 = lean_ctor_get(x_11, 1); +lean_inc(x_19); +lean_dec(x_11); +x_20 = lean_ctor_get(x_12, 0); +lean_inc(x_20); +lean_dec(x_12); +lean_inc(x_8); +x_21 = l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_19); +x_22 = lean_ctor_get(x_21, 0); +lean_inc(x_22); +if (lean_obj_tag(x_22) == 0) +{ +uint8_t x_23; +x_23 = !lean_is_exclusive(x_21); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_21, 1); +x_25 = lean_ctor_get(x_21, 0); +lean_dec(x_25); +lean_inc(x_20); +lean_ctor_set(x_21, 1, x_20); +lean_ctor_set(x_21, 0, x_20); +x_26 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5(x_1, x_21, x_4, x_5, x_6, x_7, x_8, x_9, x_24); +lean_dec(x_8); +return x_26; +} +else +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_21, 1); +lean_inc(x_27); +lean_dec(x_21); +lean_inc(x_20); +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_20); +lean_ctor_set(x_28, 1, x_20); +x_29 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5(x_1, x_28, x_4, x_5, x_6, x_7, x_8, x_9, x_27); +lean_dec(x_8); +return x_29; +} +} +else +{ +uint8_t x_30; +x_30 = !lean_is_exclusive(x_21); +if (x_30 == 0) +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_31 = lean_ctor_get(x_21, 1); +x_32 = lean_ctor_get(x_21, 0); +lean_dec(x_32); +x_33 = lean_ctor_get(x_22, 0); +lean_inc(x_33); +lean_dec(x_22); +lean_ctor_set(x_21, 1, x_33); +lean_ctor_set(x_21, 0, x_20); +x_34 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5(x_1, x_21, x_4, x_5, x_6, x_7, x_8, x_9, x_31); +lean_dec(x_8); +return x_34; +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_35 = lean_ctor_get(x_21, 1); +lean_inc(x_35); +lean_dec(x_21); +x_36 = lean_ctor_get(x_22, 0); +lean_inc(x_36); +lean_dec(x_22); +x_37 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_37, 0, x_20); +lean_ctor_set(x_37, 1, x_36); +x_38 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5(x_1, x_37, x_4, x_5, x_6, x_7, x_8, x_9, x_35); +lean_dec(x_8); +return x_38; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutErrToSorry___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; @@ -5041,7 +5077,7 @@ lean_dec(x_29); x_30 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__3___closed__1; lean_inc(x_2); x_31 = l_Lean_TagDeclarationExtension_tag(x_30, x_28, x_2); -x_32 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__2; +x_32 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__2; lean_ctor_set(x_25, 4, x_32); lean_ctor_set(x_25, 0, x_31); x_33 = lean_st_ref_set(x_11, x_25, x_26); @@ -5057,10 +5093,10 @@ lean_dec(x_35); x_38 = !lean_is_exclusive(x_36); if (x_38 == 0) { -lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; +lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; x_39 = lean_ctor_get(x_36, 1); lean_dec(x_39); -x_40 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5; +x_40 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5; lean_ctor_set(x_36, 1, x_40); x_41 = lean_st_ref_set(x_9, x_36, x_37); x_42 = lean_ctor_get(x_41, 1); @@ -5068,272 +5104,181 @@ lean_inc(x_42); lean_dec(x_41); x_43 = lean_ctor_get(x_10, 5); lean_inc(x_43); -lean_inc(x_10); -x_44 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3(x_43, x_6, x_7, x_8, x_9, x_10, x_11, x_42); -x_45 = lean_ctor_get(x_44, 0); -lean_inc(x_45); -x_46 = lean_ctor_get(x_44, 1); -lean_inc(x_46); -lean_dec(x_44); -lean_inc(x_10); -x_47 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3(x_43, x_6, x_7, x_8, x_9, x_10, x_11, x_46); -lean_dec(x_43); -x_48 = !lean_is_exclusive(x_47); -if (x_48 == 0) -{ -lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_49 = lean_ctor_get(x_47, 0); -x_50 = lean_ctor_get(x_47, 1); -lean_ctor_set(x_47, 1, x_49); -lean_ctor_set(x_47, 0, x_45); -x_51 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4(x_2, x_47, x_6, x_7, x_8, x_9, x_10, x_11, x_50); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_6); -return x_51; -} -else -{ -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_52 = lean_ctor_get(x_47, 0); -x_53 = lean_ctor_get(x_47, 1); -lean_inc(x_53); -lean_inc(x_52); -lean_dec(x_47); -x_54 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_54, 0, x_45); -lean_ctor_set(x_54, 1, x_52); -x_55 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4(x_2, x_54, x_6, x_7, x_8, x_9, x_10, x_11, x_53); +x_44 = lean_box(0); +x_45 = l_Lean_Elab_addDeclarationRangesFromSyntax___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3(x_2, x_43, x_44, x_6, x_7, x_8, x_9, x_10, x_11, x_42); lean_dec(x_11); -lean_dec(x_10); lean_dec(x_6); -return x_55; -} -} -else -{ -lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_56 = lean_ctor_get(x_36, 0); -x_57 = lean_ctor_get(x_36, 2); -x_58 = lean_ctor_get(x_36, 3); -x_59 = lean_ctor_get(x_36, 4); -lean_inc(x_59); -lean_inc(x_58); -lean_inc(x_57); -lean_inc(x_56); -lean_dec(x_36); -x_60 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5; -x_61 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_61, 0, x_56); -lean_ctor_set(x_61, 1, x_60); -lean_ctor_set(x_61, 2, x_57); -lean_ctor_set(x_61, 3, x_58); -lean_ctor_set(x_61, 4, x_59); -x_62 = lean_st_ref_set(x_9, x_61, x_37); -x_63 = lean_ctor_get(x_62, 1); -lean_inc(x_63); -lean_dec(x_62); -x_64 = lean_ctor_get(x_10, 5); -lean_inc(x_64); -lean_inc(x_10); -x_65 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3(x_64, x_6, x_7, x_8, x_9, x_10, x_11, x_63); -x_66 = lean_ctor_get(x_65, 0); -lean_inc(x_66); -x_67 = lean_ctor_get(x_65, 1); -lean_inc(x_67); -lean_dec(x_65); -lean_inc(x_10); -x_68 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3(x_64, x_6, x_7, x_8, x_9, x_10, x_11, x_67); -lean_dec(x_64); -x_69 = lean_ctor_get(x_68, 0); -lean_inc(x_69); -x_70 = lean_ctor_get(x_68, 1); -lean_inc(x_70); -if (lean_is_exclusive(x_68)) { - lean_ctor_release(x_68, 0); - lean_ctor_release(x_68, 1); - x_71 = x_68; -} else { - lean_dec_ref(x_68); - x_71 = lean_box(0); -} -if (lean_is_scalar(x_71)) { - x_72 = lean_alloc_ctor(0, 2, 0); -} else { - x_72 = x_71; +lean_dec(x_43); +return x_45; } -lean_ctor_set(x_72, 0, x_66); -lean_ctor_set(x_72, 1, x_69); -x_73 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4(x_2, x_72, x_6, x_7, x_8, x_9, x_10, x_11, x_70); +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_ctor_get(x_36, 0); +x_47 = lean_ctor_get(x_36, 2); +x_48 = lean_ctor_get(x_36, 3); +x_49 = lean_ctor_get(x_36, 4); +lean_inc(x_49); +lean_inc(x_48); +lean_inc(x_47); +lean_inc(x_46); +lean_dec(x_36); +x_50 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5; +x_51 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_51, 0, x_46); +lean_ctor_set(x_51, 1, x_50); +lean_ctor_set(x_51, 2, x_47); +lean_ctor_set(x_51, 3, x_48); +lean_ctor_set(x_51, 4, x_49); +x_52 = lean_st_ref_set(x_9, x_51, x_37); +x_53 = lean_ctor_get(x_52, 1); +lean_inc(x_53); +lean_dec(x_52); +x_54 = lean_ctor_get(x_10, 5); +lean_inc(x_54); +x_55 = lean_box(0); +x_56 = l_Lean_Elab_addDeclarationRangesFromSyntax___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3(x_2, x_54, x_55, x_6, x_7, x_8, x_9, x_10, x_11, x_53); lean_dec(x_11); -lean_dec(x_10); lean_dec(x_6); -return x_73; +lean_dec(x_54); +return x_56; } } else { -lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; -x_74 = lean_ctor_get(x_25, 0); -x_75 = lean_ctor_get(x_25, 1); -x_76 = lean_ctor_get(x_25, 2); -x_77 = lean_ctor_get(x_25, 3); -x_78 = lean_ctor_get(x_25, 5); -x_79 = lean_ctor_get(x_25, 6); -lean_inc(x_79); -lean_inc(x_78); -lean_inc(x_77); -lean_inc(x_76); -lean_inc(x_75); -lean_inc(x_74); +lean_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; +x_57 = lean_ctor_get(x_25, 0); +x_58 = lean_ctor_get(x_25, 1); +x_59 = lean_ctor_get(x_25, 2); +x_60 = lean_ctor_get(x_25, 3); +x_61 = lean_ctor_get(x_25, 5); +x_62 = lean_ctor_get(x_25, 6); +lean_inc(x_62); +lean_inc(x_61); +lean_inc(x_60); +lean_inc(x_59); +lean_inc(x_58); +lean_inc(x_57); lean_dec(x_25); -x_80 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__3___closed__1; +x_63 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__3___closed__1; lean_inc(x_2); -x_81 = l_Lean_TagDeclarationExtension_tag(x_80, x_74, x_2); -x_82 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__2; -x_83 = lean_alloc_ctor(0, 7, 0); -lean_ctor_set(x_83, 0, x_81); -lean_ctor_set(x_83, 1, x_75); -lean_ctor_set(x_83, 2, x_76); -lean_ctor_set(x_83, 3, x_77); -lean_ctor_set(x_83, 4, x_82); -lean_ctor_set(x_83, 5, x_78); -lean_ctor_set(x_83, 6, x_79); -x_84 = lean_st_ref_set(x_11, x_83, x_26); -x_85 = lean_ctor_get(x_84, 1); -lean_inc(x_85); -lean_dec(x_84); -x_86 = lean_st_ref_take(x_9, x_85); -x_87 = lean_ctor_get(x_86, 0); -lean_inc(x_87); -x_88 = lean_ctor_get(x_86, 1); -lean_inc(x_88); -lean_dec(x_86); -x_89 = lean_ctor_get(x_87, 0); -lean_inc(x_89); -x_90 = lean_ctor_get(x_87, 2); -lean_inc(x_90); -x_91 = lean_ctor_get(x_87, 3); -lean_inc(x_91); -x_92 = lean_ctor_get(x_87, 4); -lean_inc(x_92); -if (lean_is_exclusive(x_87)) { - lean_ctor_release(x_87, 0); - lean_ctor_release(x_87, 1); - lean_ctor_release(x_87, 2); - lean_ctor_release(x_87, 3); - lean_ctor_release(x_87, 4); - x_93 = x_87; -} else { - lean_dec_ref(x_87); - x_93 = lean_box(0); -} -x_94 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5; -if (lean_is_scalar(x_93)) { - x_95 = lean_alloc_ctor(0, 5, 0); -} else { - x_95 = x_93; -} -lean_ctor_set(x_95, 0, x_89); -lean_ctor_set(x_95, 1, x_94); -lean_ctor_set(x_95, 2, x_90); -lean_ctor_set(x_95, 3, x_91); -lean_ctor_set(x_95, 4, x_92); -x_96 = lean_st_ref_set(x_9, x_95, x_88); -x_97 = lean_ctor_get(x_96, 1); -lean_inc(x_97); -lean_dec(x_96); -x_98 = lean_ctor_get(x_10, 5); -lean_inc(x_98); -lean_inc(x_10); -x_99 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3(x_98, x_6, x_7, x_8, x_9, x_10, x_11, x_97); -x_100 = lean_ctor_get(x_99, 0); -lean_inc(x_100); -x_101 = lean_ctor_get(x_99, 1); -lean_inc(x_101); -lean_dec(x_99); -lean_inc(x_10); -x_102 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3(x_98, x_6, x_7, x_8, x_9, x_10, x_11, x_101); -lean_dec(x_98); -x_103 = lean_ctor_get(x_102, 0); -lean_inc(x_103); -x_104 = lean_ctor_get(x_102, 1); -lean_inc(x_104); -if (lean_is_exclusive(x_102)) { - lean_ctor_release(x_102, 0); - lean_ctor_release(x_102, 1); - x_105 = x_102; +x_64 = l_Lean_TagDeclarationExtension_tag(x_63, x_57, x_2); +x_65 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__2; +x_66 = lean_alloc_ctor(0, 7, 0); +lean_ctor_set(x_66, 0, x_64); +lean_ctor_set(x_66, 1, x_58); +lean_ctor_set(x_66, 2, x_59); +lean_ctor_set(x_66, 3, x_60); +lean_ctor_set(x_66, 4, x_65); +lean_ctor_set(x_66, 5, x_61); +lean_ctor_set(x_66, 6, x_62); +x_67 = lean_st_ref_set(x_11, x_66, x_26); +x_68 = lean_ctor_get(x_67, 1); +lean_inc(x_68); +lean_dec(x_67); +x_69 = lean_st_ref_take(x_9, x_68); +x_70 = lean_ctor_get(x_69, 0); +lean_inc(x_70); +x_71 = lean_ctor_get(x_69, 1); +lean_inc(x_71); +lean_dec(x_69); +x_72 = lean_ctor_get(x_70, 0); +lean_inc(x_72); +x_73 = lean_ctor_get(x_70, 2); +lean_inc(x_73); +x_74 = lean_ctor_get(x_70, 3); +lean_inc(x_74); +x_75 = lean_ctor_get(x_70, 4); +lean_inc(x_75); +if (lean_is_exclusive(x_70)) { + lean_ctor_release(x_70, 0); + lean_ctor_release(x_70, 1); + lean_ctor_release(x_70, 2); + lean_ctor_release(x_70, 3); + lean_ctor_release(x_70, 4); + x_76 = x_70; } else { - lean_dec_ref(x_102); - x_105 = lean_box(0); + lean_dec_ref(x_70); + x_76 = lean_box(0); } -if (lean_is_scalar(x_105)) { - x_106 = lean_alloc_ctor(0, 2, 0); +x_77 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5; +if (lean_is_scalar(x_76)) { + x_78 = lean_alloc_ctor(0, 5, 0); } else { - x_106 = x_105; -} -lean_ctor_set(x_106, 0, x_100); -lean_ctor_set(x_106, 1, x_103); -x_107 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4(x_2, x_106, x_6, x_7, x_8, x_9, x_10, x_11, x_104); + x_78 = x_76; +} +lean_ctor_set(x_78, 0, x_72); +lean_ctor_set(x_78, 1, x_77); +lean_ctor_set(x_78, 2, x_73); +lean_ctor_set(x_78, 3, x_74); +lean_ctor_set(x_78, 4, x_75); +x_79 = lean_st_ref_set(x_9, x_78, x_71); +x_80 = lean_ctor_get(x_79, 1); +lean_inc(x_80); +lean_dec(x_79); +x_81 = lean_ctor_get(x_10, 5); +lean_inc(x_81); +x_82 = lean_box(0); +x_83 = l_Lean_Elab_addDeclarationRangesFromSyntax___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3(x_2, x_81, x_82, x_6, x_7, x_8, x_9, x_10, x_11, x_80); lean_dec(x_11); -lean_dec(x_10); lean_dec(x_6); -return x_107; +lean_dec(x_81); +return x_83; } } else { -uint8_t x_108; +uint8_t x_84; lean_dec(x_11); lean_dec(x_10); lean_dec(x_6); lean_dec(x_2); -x_108 = !lean_is_exclusive(x_22); -if (x_108 == 0) +x_84 = !lean_is_exclusive(x_22); +if (x_84 == 0) { return x_22; } else { -lean_object* x_109; lean_object* x_110; lean_object* x_111; -x_109 = lean_ctor_get(x_22, 0); -x_110 = lean_ctor_get(x_22, 1); -lean_inc(x_110); -lean_inc(x_109); +lean_object* x_85; lean_object* x_86; lean_object* x_87; +x_85 = lean_ctor_get(x_22, 0); +x_86 = lean_ctor_get(x_22, 1); +lean_inc(x_86); +lean_inc(x_85); lean_dec(x_22); -x_111 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_111, 0, x_109); -lean_ctor_set(x_111, 1, x_110); -return x_111; +x_87 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_87, 0, x_85); +lean_ctor_set(x_87, 1, x_86); +return x_87; } } } else { -uint8_t x_112; +uint8_t x_88; lean_dec(x_11); lean_dec(x_10); lean_dec(x_6); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_112 = !lean_is_exclusive(x_13); -if (x_112 == 0) +x_88 = !lean_is_exclusive(x_13); +if (x_88 == 0) { return x_13; } else { -lean_object* x_113; lean_object* x_114; lean_object* x_115; -x_113 = lean_ctor_get(x_13, 0); -x_114 = lean_ctor_get(x_13, 1); -lean_inc(x_114); -lean_inc(x_113); +lean_object* x_89; lean_object* x_90; lean_object* x_91; +x_89 = lean_ctor_get(x_13, 0); +x_90 = lean_ctor_get(x_13, 1); +lean_inc(x_90); +lean_inc(x_89); lean_dec(x_13); -x_115 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_115, 0, x_113); -lean_ctor_set(x_115, 1, x_114); -return x_115; +x_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; } } } @@ -5658,7 +5603,7 @@ lean_inc(x_8); x_17 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withDeclName___rarg), 9, 2); lean_closure_set(x_17, 0, x_8); lean_closure_set(x_17, 1, x_16); -x_18 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withoutErrToSorry___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5), 8, 1); +x_18 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withoutErrToSorry___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__6), 8, 1); lean_closure_set(x_18, 0, x_17); x_19 = l_Lean_Elab_Command_liftTermElabM___rarg(x_18, x_4, x_5, x_12); if (lean_obj_tag(x_19) == 0) @@ -5844,7 +5789,7 @@ lean_inc(x_8); x_66 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withDeclName___rarg), 9, 2); lean_closure_set(x_66, 0, x_8); lean_closure_set(x_66, 1, x_65); -x_67 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withoutErrToSorry___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5), 8, 1); +x_67 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withoutErrToSorry___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__6), 8, 1); lean_closure_set(x_67, 0, x_66); x_68 = l_Lean_Elab_Command_liftTermElabM___rarg(x_67, x_4, x_5, x_61); if (lean_obj_tag(x_68) == 0) @@ -6006,7 +5951,7 @@ x_14 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___closed__2; x_15 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_15, 0, x_6); lean_ctor_set(x_15, 1, x_14); -x_16 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_15, x_3, x_4, x_9); +x_16 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__7(x_15, x_3, x_4, x_9); x_17 = !lean_is_exclusive(x_16); if (x_17 == 0) { @@ -6061,7 +6006,7 @@ x_30 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___closed__2; x_31 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_31, 0, x_29); lean_ctor_set(x_31, 1, x_30); -x_32 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_31, x_3, x_4, x_24); +x_32 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__7(x_31, x_3, x_4, x_24); x_33 = lean_ctor_get(x_32, 0); lean_inc(x_33); x_34 = lean_ctor_get(x_32, 1); @@ -6119,11 +6064,11 @@ lean_dec(x_3); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; -x_9 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_7); lean_dec(x_5); lean_dec(x_4); @@ -6133,74 +6078,286 @@ lean_dec(x_1); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRangesFromSyntax___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_Elab_addDeclarationRangesFromSyntax___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; +x_6 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__1(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; +x_13 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_5); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___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: +{ +uint8_t x_11; lean_object* x_12; +x_11 = lean_unbox(x_2); +lean_dec(x_2); +x_12 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__4(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_Lean_Elab_Tactic_Ext_realizeExtTheorem___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) { +_start: +{ +uint8_t x_7; lean_object* x_8; +x_7 = lean_unbox(x_2); +lean_dec(x_2); +x_8 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__5(x_1, x_7, x_3, x_4, x_5, x_6); +lean_dec(x_5); +lean_dec(x_3); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___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_Elab_Tactic_Ext_realizeExtTheorem(x_1, x_6, x_3, x_4, x_5); +lean_dec(x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___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; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_5 = l_Lean_Elab_Command_getRef(x_2, x_3, x_4); +x_6 = lean_ctor_get(x_5, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_5, 1); +lean_inc(x_7); +lean_dec(x_5); +x_8 = lean_ctor_get(x_2, 4); +lean_inc(x_8); +lean_inc(x_8); +x_9 = l_Lean_Elab_getBetterRef(x_6, x_8); +lean_dec(x_6); +x_10 = l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1(x_1, x_2, x_3, x_7); +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_12 = lean_ctor_get(x_10, 0); +x_13 = lean_ctor_get(x_10, 1); +x_14 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_12, x_8, x_2, x_3, x_13); +lean_dec(x_2); +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 0) +{ +lean_object* x_16; +x_16 = lean_ctor_get(x_14, 0); +lean_ctor_set(x_10, 1, x_16); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set_tag(x_14, 1); +lean_ctor_set(x_14, 0, x_10); +return x_14; +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_14, 0); +x_18 = lean_ctor_get(x_14, 1); +lean_inc(x_18); +lean_inc(x_17); +lean_dec(x_14); +lean_ctor_set(x_10, 1, x_17); +lean_ctor_set(x_10, 0, x_9); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_10); +lean_ctor_set(x_19, 1, 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; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_20 = lean_ctor_get(x_10, 0); +x_21 = lean_ctor_get(x_10, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_10); +x_22 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_20, x_8, x_2, x_3, x_21); +lean_dec(x_2); +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +if (lean_is_exclusive(x_22)) { + lean_ctor_release(x_22, 0); + lean_ctor_release(x_22, 1); + x_25 = x_22; +} else { + lean_dec_ref(x_22); + x_25 = lean_box(0); +} +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_9); +lean_ctor_set(x_26, 1, x_23); +if (lean_is_scalar(x_25)) { + x_27 = lean_alloc_ctor(1, 2, 0); +} else { + x_27 = x_25; + lean_ctor_set_tag(x_27, 1); +} +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_24); +return x_27; +} +} +} +static lean_object* _init_l_Lean_getConstInfo___at_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___spec__1___closed__1() { _start: { -lean_object* x_10; -x_10 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -return x_10; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("unknown constant '", 18, 18); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +static lean_object* _init_l_Lean_getConstInfo___at_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___spec__1___closed__2() { _start: { -lean_object* x_6; -x_6 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__1(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_6; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_getConstInfo___at_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___spec__1___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_13; -x_13 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_9); -lean_dec(x_8); +lean_object* x_5; uint8_t x_6; +x_5 = lean_st_ref_get(x_3, x_4); +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; +x_7 = lean_ctor_get(x_5, 0); +x_8 = lean_ctor_get(x_5, 1); +x_9 = lean_ctor_get(x_7, 0); +lean_inc(x_9); lean_dec(x_7); -lean_dec(x_5); -return x_13; -} +lean_inc(x_1); +x_10 = lean_environment_find(x_9, x_1); +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; +lean_free_object(x_5); +x_11 = lean_box(0); +x_12 = l_Lean_Expr_const___override(x_1, x_11); +x_13 = l_Lean_MessageData_ofExpr(x_12); +x_14 = l_Lean_getConstInfo___at_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___spec__1___closed__2; +x_15 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_13); +x_16 = l_Lean_getConstInfoInduct___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__1___closed__2; +x_17 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_17, 0, x_15); +lean_ctor_set(x_17, 1, x_16); +x_18 = l_Lean_throwError___at_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___spec__2(x_17, x_2, x_3, x_8); +return x_18; } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___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: +else { -uint8_t x_11; lean_object* x_12; -x_11 = lean_unbox(x_2); +lean_object* x_19; lean_dec(x_2); -x_12 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__4(x_1, x_11, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_12; +lean_dec(x_1); +x_19 = lean_ctor_get(x_10, 0); +lean_inc(x_19); +lean_dec(x_10); +lean_ctor_set(x_5, 0, x_19); +return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___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) { -_start: +else { -uint8_t x_7; lean_object* x_8; -x_7 = lean_unbox(x_2); -lean_dec(x_2); -x_8 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__5(x_1, x_7, x_3, x_4, x_5, x_6); +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_20 = lean_ctor_get(x_5, 0); +x_21 = lean_ctor_get(x_5, 1); +lean_inc(x_21); +lean_inc(x_20); lean_dec(x_5); -lean_dec(x_3); -return x_8; -} +x_22 = lean_ctor_get(x_20, 0); +lean_inc(x_22); +lean_dec(x_20); +lean_inc(x_1); +x_23 = lean_environment_find(x_22, x_1); +if (lean_obj_tag(x_23) == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_24 = lean_box(0); +x_25 = l_Lean_Expr_const___override(x_1, x_24); +x_26 = l_Lean_MessageData_ofExpr(x_25); +x_27 = l_Lean_getConstInfo___at_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___spec__1___closed__2; +x_28 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_26); +x_29 = l_Lean_getConstInfoInduct___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__1___closed__2; +x_30 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +x_31 = l_Lean_throwError___at_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___spec__2(x_30, x_2, x_3, x_21); +return x_31; } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___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_32; lean_object* x_33; lean_dec(x_2); -x_7 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem(x_1, x_6, x_3, x_4, x_5); -lean_dec(x_4); -return x_7; +lean_dec(x_1); +x_32 = lean_ctor_get(x_23, 0); +lean_inc(x_32); +lean_dec(x_23); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_21); +return x_33; +} +} } } static lean_object* _init_l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__1() { @@ -7529,267 +7686,234 @@ return x_356; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +lean_object* x_10; lean_object* x_11; lean_object* x_12; x_10 = lean_ctor_get(x_7, 5); lean_inc(x_10); -lean_inc(x_7); -x_11 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3(x_10, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); -x_13 = lean_ctor_get(x_11, 1); -lean_inc(x_13); -lean_dec(x_11); -lean_inc(x_7); -x_14 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3(x_10, x_3, x_4, x_5, x_6, x_7, x_8, x_13); +x_11 = lean_box(0); +x_12 = l_Lean_Elab_addDeclarationRangesFromSyntax___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3(x_1, x_10, x_11, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_10); -x_15 = !lean_is_exclusive(x_14); -if (x_15 == 0) -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_14, 0); -x_17 = lean_ctor_get(x_14, 1); -lean_ctor_set(x_14, 1, x_16); -lean_ctor_set(x_14, 0, x_12); -x_18 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4(x_1, x_14, x_3, x_4, x_5, x_6, x_7, x_8, x_17); -lean_dec(x_7); -return x_18; -} -else -{ -lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_19 = lean_ctor_get(x_14, 0); -x_20 = lean_ctor_get(x_14, 1); -lean_inc(x_20); -lean_inc(x_19); -lean_dec(x_14); -x_21 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_21, 0, x_12); -lean_ctor_set(x_21, 1, x_19); -x_22 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4(x_1, x_21, x_3, x_4, x_5, x_6, x_7, x_8, x_20); -lean_dec(x_7); -return x_22; -} +return x_12; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_13 = l_Lean_ConstantInfo_levelParams(x_1); +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_14 = l_Lean_ConstantInfo_levelParams(x_1); lean_inc(x_2); -x_14 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_14, 0, x_2); -lean_ctor_set(x_14, 1, x_13); -lean_ctor_set(x_14, 2, x_3); -x_15 = lean_box(0); +x_15 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_15, 0, x_2); +lean_ctor_set(x_15, 1, x_14); +lean_ctor_set(x_15, 2, x_3); +x_16 = lean_box(0); lean_inc(x_2); -x_16 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_16, 0, x_2); -lean_ctor_set(x_16, 1, x_15); -x_17 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_17, 0, x_14); -lean_ctor_set(x_17, 1, x_4); -lean_ctor_set(x_17, 2, x_16); -x_18 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_18, 0, x_17); +x_17 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_17, 0, x_2); +lean_ctor_set(x_17, 1, x_16); +x_18 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_18, 0, x_15); +lean_ctor_set(x_18, 1, x_4); +lean_ctor_set(x_18, 2, x_17); +x_19 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_19, 0, x_18); +lean_inc(x_12); lean_inc(x_11); -lean_inc(x_10); -x_19 = l_Lean_addDecl(x_18, x_10, x_11, x_12); -if (lean_obj_tag(x_19) == 0) +x_20 = l_Lean_addDecl(x_19, x_11, x_12, x_13); +if (lean_obj_tag(x_20) == 0) { -lean_object* x_20; uint8_t x_21; -x_20 = lean_ctor_get(x_19, 1); -lean_inc(x_20); -lean_dec(x_19); -x_21 = l_Lean_Name_isAtomic(x_2); -if (x_21 == 0) +lean_object* x_21; uint8_t x_22; +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +x_22 = l_Lean_Name_isAtomic(x_2); +if (x_22 == 0) { -lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; -x_22 = lean_st_ref_take(x_11, x_20); -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -x_24 = lean_ctor_get(x_22, 1); +lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; +x_23 = lean_st_ref_take(x_12, x_21); +x_24 = lean_ctor_get(x_23, 0); lean_inc(x_24); -lean_dec(x_22); -x_25 = !lean_is_exclusive(x_23); -if (x_25 == 0) +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +x_26 = !lean_is_exclusive(x_24); +if (x_26 == 0) { -lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; -x_26 = lean_ctor_get(x_23, 0); -x_27 = lean_ctor_get(x_23, 4); -lean_dec(x_27); -x_28 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__3___closed__1; -lean_inc(x_2); -x_29 = l_Lean_TagDeclarationExtension_tag(x_28, x_26, x_2); -x_30 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__2; -lean_ctor_set(x_23, 4, x_30); -lean_ctor_set(x_23, 0, x_29); -x_31 = lean_st_ref_set(x_11, x_23, x_24); -x_32 = lean_ctor_get(x_31, 1); -lean_inc(x_32); -lean_dec(x_31); -x_33 = lean_st_ref_take(x_9, x_32); -x_34 = lean_ctor_get(x_33, 0); -lean_inc(x_34); -x_35 = lean_ctor_get(x_33, 1); +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; +x_27 = lean_ctor_get(x_24, 0); +x_28 = lean_ctor_get(x_24, 4); +lean_dec(x_28); +x_29 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__3___closed__1; +x_30 = l_Lean_TagDeclarationExtension_tag(x_29, x_27, x_2); +x_31 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__2; +lean_ctor_set(x_24, 4, x_31); +lean_ctor_set(x_24, 0, x_30); +x_32 = lean_st_ref_set(x_12, x_24, x_25); +x_33 = lean_ctor_get(x_32, 1); +lean_inc(x_33); +lean_dec(x_32); +x_34 = lean_st_ref_take(x_10, x_33); +x_35 = lean_ctor_get(x_34, 0); lean_inc(x_35); -lean_dec(x_33); -x_36 = !lean_is_exclusive(x_34); -if (x_36 == 0) +x_36 = lean_ctor_get(x_34, 1); +lean_inc(x_36); +lean_dec(x_34); +x_37 = !lean_is_exclusive(x_35); +if (x_37 == 0) { -lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_37 = lean_ctor_get(x_34, 1); -lean_dec(x_37); -x_38 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5; -lean_ctor_set(x_34, 1, x_38); -x_39 = lean_st_ref_set(x_9, x_34, x_35); -x_40 = lean_ctor_get(x_39, 1); -lean_inc(x_40); -lean_dec(x_39); -x_41 = lean_box(0); -x_42 = l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__2(x_2, x_41, x_6, x_7, x_8, x_9, x_10, x_11, x_40); -lean_dec(x_11); -return x_42; +lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_38 = lean_ctor_get(x_35, 1); +lean_dec(x_38); +x_39 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5; +lean_ctor_set(x_35, 1, x_39); +x_40 = lean_st_ref_set(x_10, x_35, x_36); +x_41 = lean_ctor_get(x_40, 1); +lean_inc(x_41); +lean_dec(x_40); +x_42 = lean_box(0); +x_43 = l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__2(x_5, x_42, x_7, x_8, x_9, x_10, x_11, x_12, x_41); +lean_dec(x_12); +return x_43; } else { -lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_43 = lean_ctor_get(x_34, 0); -x_44 = lean_ctor_get(x_34, 2); -x_45 = lean_ctor_get(x_34, 3); -x_46 = lean_ctor_get(x_34, 4); +lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_44 = lean_ctor_get(x_35, 0); +x_45 = lean_ctor_get(x_35, 2); +x_46 = lean_ctor_get(x_35, 3); +x_47 = lean_ctor_get(x_35, 4); +lean_inc(x_47); lean_inc(x_46); lean_inc(x_45); lean_inc(x_44); -lean_inc(x_43); -lean_dec(x_34); -x_47 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5; -x_48 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_48, 0, x_43); -lean_ctor_set(x_48, 1, x_47); -lean_ctor_set(x_48, 2, x_44); -lean_ctor_set(x_48, 3, x_45); -lean_ctor_set(x_48, 4, x_46); -x_49 = lean_st_ref_set(x_9, x_48, x_35); -x_50 = lean_ctor_get(x_49, 1); -lean_inc(x_50); -lean_dec(x_49); -x_51 = lean_box(0); -x_52 = l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__2(x_2, x_51, x_6, x_7, x_8, x_9, x_10, x_11, x_50); -lean_dec(x_11); -return x_52; +lean_dec(x_35); +x_48 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5; +x_49 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_49, 0, x_44); +lean_ctor_set(x_49, 1, x_48); +lean_ctor_set(x_49, 2, x_45); +lean_ctor_set(x_49, 3, x_46); +lean_ctor_set(x_49, 4, x_47); +x_50 = lean_st_ref_set(x_10, x_49, x_36); +x_51 = lean_ctor_get(x_50, 1); +lean_inc(x_51); +lean_dec(x_50); +x_52 = lean_box(0); +x_53 = l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__2(x_5, x_52, x_7, x_8, x_9, x_10, x_11, x_12, x_51); +lean_dec(x_12); +return x_53; } } else { -lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; -x_53 = lean_ctor_get(x_23, 0); -x_54 = lean_ctor_get(x_23, 1); -x_55 = lean_ctor_get(x_23, 2); -x_56 = lean_ctor_get(x_23, 3); -x_57 = lean_ctor_get(x_23, 5); -x_58 = lean_ctor_get(x_23, 6); +lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; +x_54 = lean_ctor_get(x_24, 0); +x_55 = lean_ctor_get(x_24, 1); +x_56 = lean_ctor_get(x_24, 2); +x_57 = lean_ctor_get(x_24, 3); +x_58 = lean_ctor_get(x_24, 5); +x_59 = lean_ctor_get(x_24, 6); +lean_inc(x_59); lean_inc(x_58); lean_inc(x_57); lean_inc(x_56); lean_inc(x_55); lean_inc(x_54); -lean_inc(x_53); -lean_dec(x_23); -x_59 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__3___closed__1; -lean_inc(x_2); -x_60 = l_Lean_TagDeclarationExtension_tag(x_59, x_53, x_2); -x_61 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__2; -x_62 = lean_alloc_ctor(0, 7, 0); -lean_ctor_set(x_62, 0, x_60); -lean_ctor_set(x_62, 1, x_54); -lean_ctor_set(x_62, 2, x_55); -lean_ctor_set(x_62, 3, x_56); -lean_ctor_set(x_62, 4, x_61); -lean_ctor_set(x_62, 5, x_57); -lean_ctor_set(x_62, 6, x_58); -x_63 = lean_st_ref_set(x_11, x_62, x_24); -x_64 = lean_ctor_get(x_63, 1); -lean_inc(x_64); -lean_dec(x_63); -x_65 = lean_st_ref_take(x_9, x_64); -x_66 = lean_ctor_get(x_65, 0); -lean_inc(x_66); -x_67 = lean_ctor_get(x_65, 1); +lean_dec(x_24); +x_60 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__3___closed__1; +x_61 = l_Lean_TagDeclarationExtension_tag(x_60, x_54, x_2); +x_62 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__2; +x_63 = lean_alloc_ctor(0, 7, 0); +lean_ctor_set(x_63, 0, x_61); +lean_ctor_set(x_63, 1, x_55); +lean_ctor_set(x_63, 2, x_56); +lean_ctor_set(x_63, 3, x_57); +lean_ctor_set(x_63, 4, x_62); +lean_ctor_set(x_63, 5, x_58); +lean_ctor_set(x_63, 6, x_59); +x_64 = lean_st_ref_set(x_12, x_63, x_25); +x_65 = lean_ctor_get(x_64, 1); +lean_inc(x_65); +lean_dec(x_64); +x_66 = lean_st_ref_take(x_10, x_65); +x_67 = lean_ctor_get(x_66, 0); lean_inc(x_67); -lean_dec(x_65); -x_68 = lean_ctor_get(x_66, 0); +x_68 = lean_ctor_get(x_66, 1); lean_inc(x_68); -x_69 = lean_ctor_get(x_66, 2); +lean_dec(x_66); +x_69 = lean_ctor_get(x_67, 0); lean_inc(x_69); -x_70 = lean_ctor_get(x_66, 3); +x_70 = lean_ctor_get(x_67, 2); lean_inc(x_70); -x_71 = lean_ctor_get(x_66, 4); +x_71 = lean_ctor_get(x_67, 3); lean_inc(x_71); -if (lean_is_exclusive(x_66)) { - lean_ctor_release(x_66, 0); - lean_ctor_release(x_66, 1); - lean_ctor_release(x_66, 2); - lean_ctor_release(x_66, 3); - lean_ctor_release(x_66, 4); - x_72 = x_66; +x_72 = lean_ctor_get(x_67, 4); +lean_inc(x_72); +if (lean_is_exclusive(x_67)) { + lean_ctor_release(x_67, 0); + lean_ctor_release(x_67, 1); + lean_ctor_release(x_67, 2); + lean_ctor_release(x_67, 3); + lean_ctor_release(x_67, 4); + x_73 = x_67; } else { - lean_dec_ref(x_66); - x_72 = lean_box(0); + lean_dec_ref(x_67); + x_73 = lean_box(0); } -x_73 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5; -if (lean_is_scalar(x_72)) { - x_74 = lean_alloc_ctor(0, 5, 0); +x_74 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5; +if (lean_is_scalar(x_73)) { + x_75 = lean_alloc_ctor(0, 5, 0); } else { - x_74 = x_72; + x_75 = x_73; } -lean_ctor_set(x_74, 0, x_68); -lean_ctor_set(x_74, 1, x_73); -lean_ctor_set(x_74, 2, x_69); -lean_ctor_set(x_74, 3, x_70); -lean_ctor_set(x_74, 4, x_71); -x_75 = lean_st_ref_set(x_9, x_74, x_67); -x_76 = lean_ctor_get(x_75, 1); -lean_inc(x_76); -lean_dec(x_75); -x_77 = lean_box(0); -x_78 = l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__2(x_2, x_77, x_6, x_7, x_8, x_9, x_10, x_11, x_76); -lean_dec(x_11); -return x_78; +lean_ctor_set(x_75, 0, x_69); +lean_ctor_set(x_75, 1, x_74); +lean_ctor_set(x_75, 2, x_70); +lean_ctor_set(x_75, 3, x_71); +lean_ctor_set(x_75, 4, x_72); +x_76 = lean_st_ref_set(x_10, x_75, x_68); +x_77 = lean_ctor_get(x_76, 1); +lean_inc(x_77); +lean_dec(x_76); +x_78 = lean_box(0); +x_79 = l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__2(x_5, x_78, x_7, x_8, x_9, x_10, x_11, x_12, x_77); +lean_dec(x_12); +return x_79; } } else { -lean_object* x_79; lean_object* x_80; -x_79 = lean_box(0); -x_80 = l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__2(x_2, x_79, x_6, x_7, x_8, x_9, x_10, x_11, x_20); -lean_dec(x_11); -return x_80; +lean_object* x_80; lean_object* x_81; +lean_dec(x_2); +x_80 = lean_box(0); +x_81 = l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__2(x_5, x_80, x_7, x_8, x_9, x_10, x_11, x_12, x_21); +lean_dec(x_12); +return x_81; } } else { -uint8_t x_81; +uint8_t x_82; +lean_dec(x_12); lean_dec(x_11); -lean_dec(x_10); +lean_dec(x_5); lean_dec(x_2); -x_81 = !lean_is_exclusive(x_19); -if (x_81 == 0) +x_82 = !lean_is_exclusive(x_20); +if (x_82 == 0) { -return x_19; +return x_20; } else { -lean_object* x_82; lean_object* x_83; lean_object* x_84; -x_82 = lean_ctor_get(x_19, 0); -x_83 = lean_ctor_get(x_19, 1); +lean_object* x_83; lean_object* x_84; lean_object* x_85; +x_83 = lean_ctor_get(x_20, 0); +x_84 = lean_ctor_get(x_20, 1); +lean_inc(x_84); lean_inc(x_83); -lean_inc(x_82); -lean_dec(x_19); -x_84 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_84, 0, x_82); -lean_ctor_set(x_84, 1, x_83); -return x_84; +lean_dec(x_20); +x_85 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_85, 0, x_83); +lean_ctor_set(x_85, 1, x_84); +return x_85; } } } @@ -7830,6 +7954,7 @@ x_13 = lean_ctor_get(x_11, 1); lean_inc(x_13); lean_dec(x_11); lean_inc(x_12); +lean_inc(x_1); x_14 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1), 9, 2); lean_closure_set(x_14, 0, x_1); lean_closure_set(x_14, 1, x_12); @@ -7862,7 +7987,7 @@ if (x_23 == 0) lean_object* x_24; lean_object* x_25; lean_free_object(x_19); x_24 = lean_box(0); -x_25 = l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__3(x_2, x_3, x_12, x_21, x_24, x_4, x_5, x_6, x_7, x_8, x_9, x_22); +x_25 = l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__3(x_2, x_3, x_12, x_21, x_1, x_24, x_4, x_5, x_6, x_7, x_8, x_9, x_22); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -7874,6 +7999,7 @@ else lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; lean_dec(x_12); lean_dec(x_3); +lean_dec(x_1); x_26 = l_Lean_MessageData_ofExpr(x_21); x_27 = l_Lean_indentD(x_26); x_28 = l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__4___closed__2; @@ -7923,7 +8049,7 @@ if (x_38 == 0) { lean_object* x_39; lean_object* x_40; x_39 = lean_box(0); -x_40 = l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__3(x_2, x_3, x_12, x_36, x_39, x_4, x_5, x_6, x_7, x_8, x_9, x_37); +x_40 = l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__3(x_2, x_3, x_12, x_36, x_1, x_39, x_4, x_5, x_6, x_7, x_8, x_9, x_37); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -7935,6 +8061,7 @@ else lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_dec(x_12); lean_dec(x_3); +lean_dec(x_1); x_41 = l_Lean_MessageData_ofExpr(x_36); x_42 = l_Lean_indentD(x_41); x_43 = l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__4___closed__2; @@ -7985,6 +8112,7 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); +lean_dec(x_1); x_52 = !lean_is_exclusive(x_16); if (x_52 == 0) { @@ -8133,7 +8261,7 @@ lean_object* x_12; lean_free_object(x_5); lean_inc(x_2); lean_inc(x_1); -x_12 = l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9(x_1, x_2, x_3, x_9); +x_12 = l_Lean_getConstInfo___at_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___spec__1(x_1, x_2, x_3, 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; lean_object* x_17; lean_object* x_18; @@ -8152,7 +8280,7 @@ lean_inc(x_6); x_16 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withDeclName___rarg), 9, 2); lean_closure_set(x_16, 0, x_6); lean_closure_set(x_16, 1, x_15); -x_17 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withoutErrToSorry___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5), 8, 1); +x_17 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withoutErrToSorry___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__6), 8, 1); lean_closure_set(x_17, 0, x_16); x_18 = l_Lean_Elab_Command_liftTermElabM___rarg(x_17, x_2, x_3, x_14); if (lean_obj_tag(x_18) == 0) @@ -8452,7 +8580,7 @@ if (x_98 == 0) lean_object* x_99; lean_inc(x_2); lean_inc(x_1); -x_99 = l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9(x_1, x_2, x_3, x_96); +x_99 = l_Lean_getConstInfo___at_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___spec__1(x_1, x_2, x_3, x_96); if (lean_obj_tag(x_99) == 0) { lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; @@ -8471,7 +8599,7 @@ lean_inc(x_6); x_103 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withDeclName___rarg), 9, 2); lean_closure_set(x_103, 0, x_6); lean_closure_set(x_103, 1, x_102); -x_104 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withoutErrToSorry___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5), 8, 1); +x_104 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withoutErrToSorry___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__6), 8, 1); lean_closure_set(x_104, 0, x_103); x_105 = l_Lean_Elab_Command_liftTermElabM___rarg(x_104, x_2, x_3, x_101); if (lean_obj_tag(x_105) == 0) @@ -8664,6 +8792,24 @@ return x_147; } } } +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___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_Elab_Tactic_Ext_realizeExtIffTheorem___spec__2(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___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_getConstInfo___at_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___spec__1(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; +} +} LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___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: { @@ -8678,18 +8824,18 @@ lean_dec(x_2); return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -lean_object* x_13; -x_13 = l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_object* x_14; +x_14 = l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); lean_dec(x_1); -return x_13; +return x_14; } } LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { @@ -8732,7 +8878,7 @@ x_1 = l_Lean_Elab_Tactic_Ext_instInhabitedExtTheorem___closed__1; return x_1; } } -LEAN_EXPORT lean_object* l_repr___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____spec__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_repr___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____spec__1(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; @@ -8741,7 +8887,7 @@ x_3 = l___private_Lean_Meta_DiscrTreeTypes_0__Lean_Meta_DiscrTree_reprKey____x40 return x_3; } } -LEAN_EXPORT lean_object* l_List_foldl___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_List_foldl___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_3) == 0) @@ -8795,7 +8941,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_Format_joinSep___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____spec__2(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_Format_joinSep___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____spec__2(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -8829,13 +8975,13 @@ lean_inc(x_8); lean_dec(x_1); x_9 = lean_unsigned_to_nat(0u); x_10 = l___private_Lean_Meta_DiscrTreeTypes_0__Lean_Meta_DiscrTree_reprKey____x40_Lean_Meta_DiscrTreeTypes___hyg_355_(x_8, x_9); -x_11 = l_List_foldl___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____spec__3(x_2, x_10, x_4); +x_11 = l_List_foldl___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____spec__3(x_2, x_10, x_4); return x_11; } } } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__1() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__1() { _start: { lean_object* x_1; @@ -8843,29 +8989,29 @@ x_1 = lean_mk_string_unchecked("declName", 8, 8); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__2() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__1; +x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__1; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__3() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__2; +x_2 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__2; x_3 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__4() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__4() { _start: { lean_object* x_1; @@ -8873,29 +9019,29 @@ x_1 = lean_mk_string_unchecked(" := ", 4, 4); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__5() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__5() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__4; +x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__4; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__6() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__3; -x_2 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__5; +x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__3; +x_2 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__5; x_3 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__7() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__7() { _start: { lean_object* x_1; lean_object* x_2; @@ -8904,7 +9050,7 @@ x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__8() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__8() { _start: { lean_object* x_1; lean_object* x_2; @@ -8914,7 +9060,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__9() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__9() { _start: { lean_object* x_1; @@ -8922,17 +9068,17 @@ x_1 = lean_mk_string_unchecked("priority", 8, 8); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__10() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__10() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__9; +x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__9; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__11() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__11() { _start: { lean_object* x_1; @@ -8940,17 +9086,17 @@ x_1 = lean_mk_string_unchecked("keys", 4, 4); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__12() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__12() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__11; +x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__11; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__13() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__13() { _start: { lean_object* x_1; lean_object* x_2; @@ -8959,7 +9105,7 @@ x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__14() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__14() { _start: { lean_object* x_1; @@ -8967,35 +9113,35 @@ x_1 = lean_mk_string_unchecked("{ ", 2, 2); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__15() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__15() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__14; +x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__14; x_2 = lean_string_length(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__16() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__16() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__15; +x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__15; x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__17() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__17() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__14; +x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__14; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__18() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__18() { _start: { lean_object* x_1; @@ -9003,21 +9149,21 @@ x_1 = lean_mk_string_unchecked(" }", 2, 2); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__19() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__19() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__18; +x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__18; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__20() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__20() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__8; +x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__8; x_2 = lean_box(1); x_3 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -9025,7 +9171,7 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__21() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__21() { _start: { lean_object* x_1; @@ -9033,35 +9179,35 @@ x_1 = lean_mk_string_unchecked("#[", 2, 2); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__22() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__22() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__21; +x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__21; x_2 = lean_string_length(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__23() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__23() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__22; +x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__22; x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__24() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__24() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__21; +x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__21; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__25() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__25() { _start: { lean_object* x_1; @@ -9069,17 +9215,17 @@ x_1 = lean_mk_string_unchecked("]", 1, 1); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__26() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__26() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__25; +x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__25; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__27() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__27() { _start: { lean_object* x_1; @@ -9087,33 +9233,33 @@ x_1 = lean_mk_string_unchecked("#[]", 3, 3); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__28() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__28() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__27; +x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__27; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__29() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__29() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__13; -x_2 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__28; +x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__13; +x_2 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__28; x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__30() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__30() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__29; +x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__29; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -9121,7 +9267,7 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191_(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085_(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; @@ -9129,7 +9275,7 @@ x_3 = lean_ctor_get(x_1, 0); lean_inc(x_3); x_4 = lean_unsigned_to_nat(0u); x_5 = l_Lean_Name_reprPrec(x_3, x_4); -x_6 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__7; +x_6 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__7; x_7 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_7, 0, x_6); lean_ctor_set(x_7, 1, x_5); @@ -9137,11 +9283,11 @@ x_8 = 0; x_9 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_9, 0, x_7); lean_ctor_set_uint8(x_9, sizeof(void*)*1, x_8); -x_10 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__6; +x_10 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__6; x_11 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_11, 0, x_10); lean_ctor_set(x_11, 1, x_9); -x_12 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__8; +x_12 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__8; x_13 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_13, 0, x_11); lean_ctor_set(x_13, 1, x_12); @@ -9149,11 +9295,11 @@ x_14 = lean_box(1); x_15 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_15, 0, x_13); lean_ctor_set(x_15, 1, x_14); -x_16 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__10; +x_16 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__10; x_17 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_17, 0, x_15); lean_ctor_set(x_17, 1, x_16); -x_18 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__5; +x_18 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__5; x_19 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_19, 0, x_17); lean_ctor_set(x_19, 1, x_18); @@ -9177,7 +9323,7 @@ lean_ctor_set(x_26, 1, x_12); x_27 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_27, 0, x_26); lean_ctor_set(x_27, 1, x_14); -x_28 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__12; +x_28 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__12; x_29 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_29, 0, x_27); lean_ctor_set(x_29, 1, x_28); @@ -9194,17 +9340,17 @@ if (x_33 == 0) { lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; x_34 = lean_array_to_list(x_31); -x_35 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__20; -x_36 = l_Std_Format_joinSep___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____spec__2(x_34, x_35); -x_37 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__24; +x_35 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__20; +x_36 = l_Std_Format_joinSep___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____spec__2(x_34, x_35); +x_37 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__24; x_38 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_38, 0, x_37); lean_ctor_set(x_38, 1, x_36); -x_39 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__26; +x_39 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__26; x_40 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_40, 0, x_38); lean_ctor_set(x_40, 1, x_39); -x_41 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__23; +x_41 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__23; x_42 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_42, 0, x_41); lean_ctor_set(x_42, 1, x_40); @@ -9212,7 +9358,7 @@ x_43 = 1; x_44 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_44, 0, x_42); lean_ctor_set_uint8(x_44, sizeof(void*)*1, x_43); -x_45 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__13; +x_45 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__13; x_46 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_46, 0, x_45); lean_ctor_set(x_46, 1, x_44); @@ -9222,15 +9368,15 @@ lean_ctor_set_uint8(x_47, sizeof(void*)*1, x_8); x_48 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_48, 0, x_30); lean_ctor_set(x_48, 1, x_47); -x_49 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__17; +x_49 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__17; x_50 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_50, 0, x_49); lean_ctor_set(x_50, 1, x_48); -x_51 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__19; +x_51 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__19; x_52 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_52, 0, x_50); lean_ctor_set(x_52, 1, x_51); -x_53 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__16; +x_53 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__16; x_54 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_54, 0, x_53); lean_ctor_set(x_54, 1, x_52); @@ -9243,19 +9389,19 @@ else { lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_dec(x_31); -x_56 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__30; +x_56 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__30; x_57 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_57, 0, x_30); lean_ctor_set(x_57, 1, x_56); -x_58 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__17; +x_58 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__17; x_59 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_59, 0, x_58); lean_ctor_set(x_59, 1, x_57); -x_60 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__19; +x_60 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__19; x_61 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_61, 0, x_59); lean_ctor_set(x_61, 1, x_60); -x_62 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__16; +x_62 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__16; x_63 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_63, 0, x_62); lean_ctor_set(x_63, 1, x_61); @@ -9266,11 +9412,11 @@ return x_64; } } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191_(x_1, x_2); +x_3 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085_(x_1, x_2); lean_dec(x_2); return x_3; } @@ -9279,7 +9425,7 @@ static lean_object* _init_l_Lean_Elab_Tactic_Ext_instReprExtTheorem___closed__1( _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____boxed), 2, 0); return x_1; } } @@ -9291,7 +9437,7 @@ x_1 = l_Lean_Elab_Tactic_Ext_instReprExtTheorem___closed__1; return x_1; } } -LEAN_EXPORT uint8_t l_Array_isEqvAux___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3269____spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT uint8_t l_Array_isEqvAux___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3163____spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; uint8_t x_9; @@ -9332,7 +9478,7 @@ return x_17; } } } -LEAN_EXPORT uint8_t l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3269_(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3163_(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; @@ -9376,18 +9522,18 @@ return x_16; else { uint8_t x_17; -x_17 = l_Array_isEqvAux___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3269____spec__1(x_5, x_8, lean_box(0), x_5, x_8, x_13, lean_box(0)); +x_17 = l_Array_isEqvAux___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3163____spec__1(x_5, x_8, lean_box(0), x_5, x_8, x_13, lean_box(0)); return x_17; } } } } } -LEAN_EXPORT lean_object* l_Array_isEqvAux___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3269____spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_isEqvAux___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3163____spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { uint8_t x_8; lean_object* x_9; -x_8 = l_Array_isEqvAux___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3269____spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Array_isEqvAux___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3163____spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); @@ -9396,11 +9542,11 @@ x_9 = lean_box(x_8); return x_9; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3269____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3163____boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3269_(x_1, x_2); +x_3 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3163_(x_1, x_2); lean_dec(x_2); lean_dec(x_1); x_4 = lean_box(x_3); @@ -9411,7 +9557,7 @@ static lean_object* _init_l_Lean_Elab_Tactic_Ext_instBEqExtTheorem___closed__1() _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3269____boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3163____boxed), 2, 0); return x_1; } } @@ -9423,7 +9569,7 @@ x_1 = l_Lean_Elab_Tactic_Ext_instBEqExtTheorem___closed__1; return x_1; } } -LEAN_EXPORT uint64_t l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3359____spec__1(lean_object* x_1, size_t x_2, size_t x_3, uint64_t x_4) { +LEAN_EXPORT uint64_t l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3253____spec__1(lean_object* x_1, size_t x_2, size_t x_3, uint64_t x_4) { _start: { uint8_t x_5; @@ -9447,7 +9593,7 @@ return x_4; } } } -LEAN_EXPORT uint64_t l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3359_(lean_object* x_1) { +LEAN_EXPORT uint64_t l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3253_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; uint64_t x_5; uint64_t x_6; uint64_t x_7; uint64_t x_8; uint64_t x_9; uint64_t x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; @@ -9487,14 +9633,14 @@ size_t x_17; size_t x_18; uint64_t x_19; uint64_t x_20; x_17 = 0; x_18 = lean_usize_of_nat(x_11); lean_dec(x_11); -x_19 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3359____spec__1(x_4, x_17, x_18, x_10); +x_19 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3253____spec__1(x_4, x_17, x_18, x_10); x_20 = lean_uint64_mix_hash(x_9, x_19); return x_20; } } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3359____spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3253____spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { size_t x_5; size_t x_6; uint64_t x_7; uint64_t x_8; lean_object* x_9; @@ -9504,17 +9650,17 @@ x_6 = lean_unbox_usize(x_3); lean_dec(x_3); x_7 = lean_unbox_uint64(x_4); lean_dec(x_4); -x_8 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3359____spec__1(x_1, x_5, x_6, x_7); +x_8 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3253____spec__1(x_1, x_5, x_6, x_7); lean_dec(x_1); x_9 = lean_box_uint64(x_8); return x_9; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3359____boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3253____boxed(lean_object* x_1) { _start: { uint64_t x_2; lean_object* x_3; -x_2 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3359_(x_1); +x_2 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3253_(x_1); lean_dec(x_1); x_3 = lean_box_uint64(x_2); return x_3; @@ -9524,7 +9670,7 @@ static lean_object* _init_l_Lean_Elab_Tactic_Ext_instHashableExtTheorem___closed _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3359____boxed), 1, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3253____boxed), 1, 0); return x_1; } } @@ -9579,7 +9725,7 @@ x_1 = l_Lean_Elab_Tactic_Ext_extExt_config___closed__1; return x_1; } } -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; uint8_t x_7; @@ -9621,7 +9767,7 @@ return x_15; } } } -static size_t _init_l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3___closed__1() { +static size_t _init_l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__3___closed__1() { _start: { size_t x_1; size_t x_2; size_t x_3; @@ -9631,17 +9777,17 @@ x_3 = lean_usize_shift_left(x_1, x_2); return x_3; } } -static size_t _init_l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3___closed__2() { +static size_t _init_l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__3___closed__2() { _start: { size_t x_1; size_t x_2; size_t x_3; x_1 = 1; -x_2 = l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3___closed__1; +x_2 = l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__3___closed__1; x_3 = lean_usize_sub(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3(lean_object* x_1, size_t x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__3(lean_object* x_1, size_t x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_1) == 0) @@ -9653,7 +9799,7 @@ if (x_4 == 0) lean_object* x_5; size_t x_6; size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; x_5 = lean_ctor_get(x_1, 0); x_6 = 5; -x_7 = l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3___closed__2; +x_7 = l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__3___closed__2; x_8 = lean_usize_land(x_2, x_7); x_9 = lean_usize_to_nat(x_8); x_10 = lean_box(2); @@ -9714,7 +9860,7 @@ x_20 = lean_ctor_get(x_1, 0); lean_inc(x_20); lean_dec(x_1); x_21 = 5; -x_22 = l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3___closed__2; +x_22 = l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__3___closed__2; x_23 = lean_usize_land(x_2, x_22); x_24 = lean_usize_to_nat(x_23); x_25 = lean_box(2); @@ -9776,24 +9922,24 @@ x_37 = lean_ctor_get(x_1, 1); lean_inc(x_37); lean_dec(x_1); x_38 = lean_unsigned_to_nat(0u); -x_39 = l_Lean_PersistentHashMap_findAtAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__4(x_36, x_37, lean_box(0), x_38, x_3); +x_39 = l_Lean_PersistentHashMap_findAtAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__4(x_36, x_37, lean_box(0), x_38, x_3); lean_dec(x_37); lean_dec(x_36); return x_39; } } } -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__2(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__2(lean_object* x_1, lean_object* x_2) { _start: { uint64_t x_3; size_t x_4; lean_object* x_5; x_3 = l_Lean_Meta_DiscrTree_Key_hash(x_2); x_4 = lean_uint64_to_usize(x_3); -x_5 = l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3(x_1, x_4, x_2); +x_5 = l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__3(x_1, x_4, x_2); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__7(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__7(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; uint8_t x_8; @@ -9820,7 +9966,7 @@ x_17 = lean_usize_shift_right(x_12, x_16); x_18 = lean_unsigned_to_nat(1u); x_19 = lean_nat_add(x_5, x_18); lean_dec(x_5); -x_20 = l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__6(x_6, x_17, x_1, x_9, x_10); +x_20 = l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__6(x_6, x_17, x_1, x_9, x_10); x_4 = lean_box(0); x_5 = x_19; x_6 = x_20; @@ -9828,7 +9974,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; @@ -9920,7 +10066,7 @@ return x_29; } } } -static lean_object* _init_l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__6___closed__1() { +static lean_object* _init_l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__6___closed__1() { _start: { lean_object* x_1; @@ -9928,7 +10074,7 @@ x_1 = l_Lean_PersistentHashMap_mkEmptyEntries(lean_box(0), lean_box(0)); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__6(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__6(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5) { _start: { if (lean_obj_tag(x_1) == 0) @@ -9941,7 +10087,7 @@ lean_object* x_7; size_t x_8; size_t x_9; size_t x_10; size_t x_11; lean_object* x_7 = lean_ctor_get(x_1, 0); x_8 = 1; x_9 = 5; -x_10 = l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3___closed__2; +x_10 = l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__3___closed__2; x_11 = lean_usize_land(x_2, x_10); x_12 = lean_usize_to_nat(x_11); x_13 = lean_array_get_size(x_7); @@ -10041,7 +10187,7 @@ lean_object* x_35; size_t x_36; size_t x_37; lean_object* x_38; lean_object* x_3 x_35 = lean_ctor_get(x_15, 0); x_36 = lean_usize_shift_right(x_2, x_9); x_37 = lean_usize_add(x_3, x_8); -x_38 = l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__6(x_35, x_36, x_37, x_4, x_5); +x_38 = l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__6(x_35, x_36, x_37, x_4, x_5); lean_ctor_set(x_15, 0, x_38); x_39 = lean_array_fset(x_17, x_12, x_15); lean_dec(x_12); @@ -10056,7 +10202,7 @@ lean_inc(x_40); lean_dec(x_15); x_41 = lean_usize_shift_right(x_2, x_9); x_42 = lean_usize_add(x_3, x_8); -x_43 = l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__6(x_40, x_41, x_42, x_4, x_5); +x_43 = l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__6(x_40, x_41, x_42, x_4, x_5); x_44 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_44, 0, x_43); x_45 = lean_array_fset(x_17, x_12, x_44); @@ -10087,7 +10233,7 @@ lean_inc(x_48); lean_dec(x_1); x_49 = 1; x_50 = 5; -x_51 = l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3___closed__2; +x_51 = l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__3___closed__2; x_52 = lean_usize_land(x_2, x_51); x_53 = lean_usize_to_nat(x_52); x_54 = lean_array_get_size(x_48); @@ -10172,7 +10318,7 @@ if (lean_is_exclusive(x_57)) { } x_73 = lean_usize_shift_right(x_2, x_50); x_74 = lean_usize_add(x_3, x_49); -x_75 = l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__6(x_71, x_73, x_74, x_4, x_5); +x_75 = l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__6(x_71, x_73, x_74, x_4, x_5); if (lean_is_scalar(x_72)) { x_76 = lean_alloc_ctor(1, 1, 0); } else { @@ -10209,7 +10355,7 @@ if (x_82 == 0) { lean_object* x_83; lean_object* x_84; size_t x_85; uint8_t x_86; x_83 = lean_unsigned_to_nat(0u); -x_84 = l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__8(x_1, x_83, x_4, x_5); +x_84 = l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__8(x_1, x_83, x_4, x_5); x_85 = 7; x_86 = lean_usize_dec_le(x_85, x_3); if (x_86 == 0) @@ -10227,8 +10373,8 @@ lean_inc(x_90); x_91 = lean_ctor_get(x_84, 1); lean_inc(x_91); lean_dec(x_84); -x_92 = l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__6___closed__1; -x_93 = l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__7(x_3, x_90, x_91, lean_box(0), x_83, x_92); +x_92 = l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__6___closed__1; +x_93 = l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__7(x_3, x_90, x_91, lean_box(0), x_83, x_92); lean_dec(x_91); lean_dec(x_90); return x_93; @@ -10255,7 +10401,7 @@ x_96 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_96, 0, x_94); lean_ctor_set(x_96, 1, x_95); x_97 = lean_unsigned_to_nat(0u); -x_98 = l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__8(x_96, x_97, x_4, x_5); +x_98 = l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__8(x_96, x_97, x_4, x_5); x_99 = 7; x_100 = lean_usize_dec_le(x_99, x_3); if (x_100 == 0) @@ -10273,8 +10419,8 @@ lean_inc(x_104); x_105 = lean_ctor_get(x_98, 1); lean_inc(x_105); lean_dec(x_98); -x_106 = l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__6___closed__1; -x_107 = l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__7(x_3, x_104, x_105, lean_box(0), x_97, x_106); +x_106 = l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__6___closed__1; +x_107 = l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__7(x_3, x_104, x_105, lean_box(0), x_97, x_106); lean_dec(x_105); lean_dec(x_104); return x_107; @@ -10292,18 +10438,18 @@ return x_98; } } } -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insert___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insert___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint64_t x_4; size_t x_5; size_t x_6; lean_object* x_7; x_4 = l_Lean_Meta_DiscrTree_Key_hash(x_2); x_5 = lean_uint64_to_usize(x_4); x_6 = 1; -x_7 = l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__6(x_1, x_5, x_6, x_2, x_3); +x_7 = l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__6(x_1, x_5, x_6, x_2, x_3); return x_7; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertVal_loop___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertVal_loop___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; uint8_t x_5; @@ -10321,7 +10467,7 @@ else { lean_object* x_7; uint8_t x_8; x_7 = lean_array_fget(x_1, x_3); -x_8 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3269_(x_2, x_7); +x_8 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3163_(x_2, x_7); lean_dec(x_7); if (x_8 == 0) { @@ -10342,7 +10488,7 @@ return x_12; } } } -LEAN_EXPORT lean_object* l___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__12(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__12(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; @@ -10395,7 +10541,7 @@ x_24 = lean_ctor_get(x_19, 0); lean_dec(x_24); x_25 = lean_unsigned_to_nat(1u); x_26 = lean_nat_add(x_3, x_25); -x_27 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9(x_1, x_2, x_26, x_23); +x_27 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__9(x_1, x_2, x_26, x_23); lean_dec(x_26); lean_ctor_set(x_19, 1, x_27); lean_ctor_set(x_19, 0, x_4); @@ -10411,7 +10557,7 @@ lean_inc(x_29); lean_dec(x_19); x_30 = lean_unsigned_to_nat(1u); x_31 = lean_nat_add(x_3, x_30); -x_32 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9(x_1, x_2, x_31, x_29); +x_32 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__9(x_1, x_2, x_31, x_29); lean_dec(x_31); x_33 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_33, 0, x_4); @@ -10462,7 +10608,7 @@ return x_43; } } } -LEAN_EXPORT lean_object* l_Array_binInsertM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__11(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_binInsertM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__11(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { uint8_t x_7; @@ -10513,7 +10659,7 @@ x_21 = lean_ctor_get(x_16, 0); lean_dec(x_21); x_22 = lean_unsigned_to_nat(1u); x_23 = lean_nat_add(x_3, x_22); -x_24 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9(x_1, x_2, x_23, x_20); +x_24 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__9(x_1, x_2, x_23, x_20); lean_dec(x_23); lean_ctor_set(x_16, 1, x_24); lean_ctor_set(x_16, 0, x_4); @@ -10528,7 +10674,7 @@ lean_inc(x_26); lean_dec(x_16); x_27 = lean_unsigned_to_nat(1u); x_28 = lean_nat_add(x_3, x_27); -x_29 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9(x_1, x_2, x_28, x_26); +x_29 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__9(x_1, x_2, x_28, x_26); lean_dec(x_28); x_30 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_30, 0, x_4); @@ -10583,7 +10729,7 @@ x_44 = lean_ctor_get(x_40, 1); x_45 = lean_ctor_get(x_40, 0); lean_dec(x_45); x_46 = lean_nat_add(x_3, x_37); -x_47 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9(x_1, x_2, x_46, x_44); +x_47 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__9(x_1, x_2, x_46, x_44); lean_dec(x_46); lean_ctor_set(x_40, 1, x_47); lean_ctor_set(x_40, 0, x_4); @@ -10598,7 +10744,7 @@ x_49 = lean_ctor_get(x_40, 1); lean_inc(x_49); lean_dec(x_40); x_50 = lean_nat_add(x_3, x_37); -x_51 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9(x_1, x_2, x_50, x_49); +x_51 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__9(x_1, x_2, x_50, x_49); lean_dec(x_50); x_52 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_52, 0, x_4); @@ -10616,7 +10762,7 @@ x_54 = lean_array_get_size(x_5); x_55 = lean_unsigned_to_nat(1u); x_56 = lean_nat_sub(x_54, x_55); lean_dec(x_54); -x_57 = l___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__12(x_1, x_2, x_3, x_4, x_5, x_6, x_8, x_56); +x_57 = l___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__12(x_1, x_2, x_3, x_4, x_5, x_6, x_8, x_56); return x_57; } } @@ -10671,7 +10817,7 @@ return x_72; } } } -static lean_object* _init_l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9___closed__1() { +static lean_object* _init_l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__9___closed__1() { _start: { lean_object* x_1; lean_object* x_2; @@ -10682,7 +10828,7 @@ lean_ctor_set(x_2, 1, x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { uint8_t x_5; @@ -10699,7 +10845,7 @@ if (x_9 == 0) { lean_object* x_10; lean_object* x_11; x_10 = lean_unsigned_to_nat(0u); -x_11 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertVal_loop___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__10(x_6, x_2, x_10); +x_11 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertVal_loop___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__10(x_6, x_2, x_10); lean_ctor_set(x_4, 0, x_11); return x_4; } @@ -10707,12 +10853,12 @@ else { lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; x_12 = lean_array_fget(x_1, x_3); -x_13 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9___closed__1; +x_13 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__9___closed__1; lean_inc(x_12); x_14 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_14, 0, x_12); lean_ctor_set(x_14, 1, x_13); -x_15 = l_Array_binInsertM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__11(x_1, x_2, x_3, x_12, x_7, x_14); +x_15 = l_Array_binInsertM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__11(x_1, x_2, x_3, x_12, x_7, x_14); lean_ctor_set(x_4, 1, x_15); return x_4; } @@ -10732,7 +10878,7 @@ if (x_19 == 0) { lean_object* x_20; lean_object* x_21; lean_object* x_22; x_20 = lean_unsigned_to_nat(0u); -x_21 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertVal_loop___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__10(x_16, x_2, x_20); +x_21 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertVal_loop___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__10(x_16, x_2, x_20); x_22 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_22, 0, x_21); lean_ctor_set(x_22, 1, x_17); @@ -10742,12 +10888,12 @@ else { lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; x_23 = lean_array_fget(x_1, x_3); -x_24 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9___closed__1; +x_24 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__9___closed__1; lean_inc(x_23); x_25 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_25, 0, x_23); lean_ctor_set(x_25, 1, x_24); -x_26 = l_Array_binInsertM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__11(x_1, x_2, x_3, x_23, x_17, x_25); +x_26 = l_Array_binInsertM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__11(x_1, x_2, x_3, x_23, x_17, x_25); x_27 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_27, 0, x_16); lean_ctor_set(x_27, 1, x_26); @@ -10756,7 +10902,7 @@ return x_27; } } } -static lean_object* _init_l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__13___closed__1() { +static lean_object* _init_l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__13___closed__1() { _start: { lean_object* x_1; @@ -10764,16 +10910,16 @@ x_1 = l_Lean_Meta_DiscrTree_instInhabited(lean_box(0)); return x_1; } } -LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__13(lean_object* x_1) { +LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__13(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__13___closed__1; +x_2 = l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__13___closed__1; x_3 = lean_panic_fn(x_2, x_1); return x_3; } } -static lean_object* _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__1() { +static lean_object* _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__1___closed__1() { _start: { lean_object* x_1; @@ -10781,7 +10927,7 @@ x_1 = lean_mk_string_unchecked("Lean.Meta.DiscrTree", 19, 19); return x_1; } } -static lean_object* _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__2() { +static lean_object* _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__1___closed__2() { _start: { lean_object* x_1; @@ -10789,7 +10935,7 @@ x_1 = lean_mk_string_unchecked("Lean.Meta.DiscrTree.insertCore", 30, 30); return x_1; } } -static lean_object* _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__3() { +static lean_object* _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__1___closed__3() { _start: { lean_object* x_1; @@ -10797,20 +10943,20 @@ x_1 = lean_mk_string_unchecked("invalid key sequence", 20, 20); return x_1; } } -static lean_object* _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__4() { +static lean_object* _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__1___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__1; -x_2 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__2; +x_1 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__1___closed__1; +x_2 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__1___closed__2; x_3 = lean_unsigned_to_nat(484u); x_4 = lean_unsigned_to_nat(23u); -x_5 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__3; +x_5 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -10828,13 +10974,13 @@ lean_object* x_8; lean_object* x_9; lean_object* x_10; x_8 = l_Lean_Meta_DiscrTree_instInhabitedKey; x_9 = l_outOfBounds___rarg(x_8); lean_inc(x_1); -x_10 = l_Lean_PersistentHashMap_find_x3f___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__2(x_1, x_9); +x_10 = l_Lean_PersistentHashMap_find_x3f___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__2(x_1, x_9); if (lean_obj_tag(x_10) == 0) { lean_object* x_11; lean_object* x_12; lean_object* x_13; x_11 = lean_unsigned_to_nat(1u); x_12 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_createNodes___rarg(x_2, x_3, x_11); -x_13 = l_Lean_PersistentHashMap_insert___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__5(x_1, x_9, x_12); +x_13 = l_Lean_PersistentHashMap_insert___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__5(x_1, x_9, x_12); return x_13; } else @@ -10844,8 +10990,8 @@ x_14 = lean_ctor_get(x_10, 0); lean_inc(x_14); lean_dec(x_10); x_15 = lean_unsigned_to_nat(1u); -x_16 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9(x_2, x_3, x_15, x_14); -x_17 = l_Lean_PersistentHashMap_insert___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__5(x_1, x_9, x_16); +x_16 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__9(x_2, x_3, x_15, x_14); +x_17 = l_Lean_PersistentHashMap_insert___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__5(x_1, x_9, x_16); return x_17; } } @@ -10854,13 +11000,13 @@ else lean_object* x_18; lean_object* x_19; x_18 = lean_array_fget(x_2, x_6); lean_inc(x_1); -x_19 = l_Lean_PersistentHashMap_find_x3f___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__2(x_1, x_18); +x_19 = l_Lean_PersistentHashMap_find_x3f___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__2(x_1, x_18); if (lean_obj_tag(x_19) == 0) { lean_object* x_20; lean_object* x_21; lean_object* x_22; x_20 = lean_unsigned_to_nat(1u); x_21 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_createNodes___rarg(x_2, x_3, x_20); -x_22 = l_Lean_PersistentHashMap_insert___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__5(x_1, x_18, x_21); +x_22 = l_Lean_PersistentHashMap_insert___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__5(x_1, x_18, x_21); return x_22; } else @@ -10870,8 +11016,8 @@ x_23 = lean_ctor_get(x_19, 0); lean_inc(x_23); lean_dec(x_19); x_24 = lean_unsigned_to_nat(1u); -x_25 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9(x_2, x_3, x_24, x_23); -x_26 = l_Lean_PersistentHashMap_insert___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__5(x_1, x_18, x_25); +x_25 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__9(x_2, x_3, x_24, x_23); +x_26 = l_Lean_PersistentHashMap_insert___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__5(x_1, x_18, x_25); return x_26; } } @@ -10881,13 +11027,13 @@ else lean_object* x_27; lean_object* x_28; lean_dec(x_3); lean_dec(x_1); -x_27 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__4; -x_28 = l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__13(x_27); +x_27 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__1___closed__4; +x_28 = l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__13(x_27); return x_28; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____lambda__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____lambda__1(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; @@ -10900,7 +11046,7 @@ x_5 = lean_ctor_get(x_1, 1); x_6 = lean_ctor_get(x_2, 2); lean_inc(x_6); lean_inc(x_2); -x_7 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1(x_4, x_6, x_2); +x_7 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__1(x_4, x_6, x_2); lean_dec(x_6); x_8 = lean_ctor_get(x_2, 0); lean_inc(x_8); @@ -10922,7 +11068,7 @@ lean_dec(x_1); x_12 = lean_ctor_get(x_2, 2); lean_inc(x_12); lean_inc(x_2); -x_13 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1(x_10, x_12, x_2); +x_13 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__1(x_10, x_12, x_2); lean_dec(x_12); x_14 = lean_ctor_get(x_2, 0); lean_inc(x_14); @@ -10936,7 +11082,7 @@ return x_16; } } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__1() { _start: { lean_object* x_1; @@ -10944,7 +11090,7 @@ x_1 = lean_mk_string_unchecked("Elab", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__2() { _start: { lean_object* x_1; @@ -10952,7 +11098,7 @@ x_1 = lean_mk_string_unchecked("Ext", 3, 3); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__3() { _start: { lean_object* x_1; @@ -10960,28 +11106,28 @@ x_1 = lean_mk_string_unchecked("extExtension", 12, 12); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__1; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__1; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__1; x_3 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__10; -x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__2; -x_5 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__3; +x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__2; +x_5 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__3; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__5() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____lambda__1), 2, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____lambda__1), 2, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__6() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__6() { _start: { lean_object* x_1; @@ -10989,14 +11135,14 @@ x_1 = lean_alloc_closure((void*)(l_id___rarg___boxed), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__7() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__4; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__5; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__4; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__5; x_3 = l_Lean_Elab_Tactic_Ext_instInhabitedExtTheorems___closed__1; -x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__6; +x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__6; x_5 = lean_alloc_ctor(0, 4, 0); lean_ctor_set(x_5, 0, x_1); lean_ctor_set(x_5, 1, x_2); @@ -11005,59 +11151,59 @@ lean_ctor_set(x_5, 3, x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__7; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__7; x_3 = l_Lean_registerSimpleScopedEnvExtension___rarg(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; -x_6 = l_Lean_PersistentHashMap_findAtAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__4(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Lean_PersistentHashMap_findAtAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__4(x_1, x_2, x_3, x_4, x_5); lean_dec(x_5); lean_dec(x_2); lean_dec(x_1); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { size_t x_4; lean_object* x_5; x_4 = lean_unbox_usize(x_2); lean_dec(x_2); -x_5 = l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3(x_1, x_4, x_3); +x_5 = l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__3(x_1, x_4, x_3); lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__2___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__2___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Lean_PersistentHashMap_find_x3f___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__2(x_1, x_2); +x_3 = l_Lean_PersistentHashMap_find_x3f___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__2(x_1, x_2); lean_dec(x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { size_t x_7; lean_object* x_8; x_7 = lean_unbox_usize(x_1); lean_dec(x_1); -x_8 = l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__7(x_7, x_2, x_3, x_4, x_5, x_6); +x_8 = l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__7(x_7, x_2, x_3, x_4, x_5, x_6); lean_dec(x_3); lean_dec(x_2); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { size_t x_6; size_t x_7; lean_object* x_8; @@ -11065,45 +11211,45 @@ x_6 = lean_unbox_usize(x_2); lean_dec(x_2); x_7 = lean_unbox_usize(x_3); lean_dec(x_3); -x_8 = l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__6(x_1, x_6, x_7, x_4, x_5); +x_8 = l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__6(x_1, x_6, x_7, x_4, x_5); return x_8; } } -LEAN_EXPORT lean_object* l___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__12___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__12___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; -x_9 = l___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__12(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__12(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_3); lean_dec(x_1); return x_9; } } -LEAN_EXPORT lean_object* l_Array_binInsertM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_binInsertM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; -x_7 = l_Array_binInsertM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__11(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Array_binInsertM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__11(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_3); lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9(x_1, x_2, x_3, x_4); +x_5 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__9(x_1, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_1); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1(x_1, x_2, x_3); +x_4 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__1(x_1, x_2, x_3); lean_dec(x_2); return x_4; } @@ -11980,7 +12126,7 @@ x_7 = lean_box(x_6); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; @@ -12068,7 +12214,7 @@ return x_27; } } } -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; @@ -12087,7 +12233,7 @@ lean_object* x_11; lean_object* x_12; x_11 = lean_ctor_get(x_3, 6); lean_dec(x_11); lean_ctor_set(x_3, 6, x_9); -x_12 = l_Lean_throwError___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__3(x_2, x_3, x_4, x_8); +x_12 = l_Lean_throwError___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__3(x_2, x_3, x_4, x_8); return x_12; } else @@ -12125,12 +12271,12 @@ lean_ctor_set(x_23, 7, x_19); lean_ctor_set(x_23, 8, x_20); lean_ctor_set(x_23, 9, x_21); lean_ctor_set_uint8(x_23, sizeof(void*)*10, x_22); -x_24 = l_Lean_throwError___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__3(x_2, x_23, x_4, x_8); +x_24 = l_Lean_throwError___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__3(x_2, x_23, x_4, x_8); return x_24; } } } -static lean_object* _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__1() { +static lean_object* _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__1() { _start: { lean_object* x_1; @@ -12138,7 +12284,7 @@ x_1 = lean_mk_string_unchecked("runtime", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__2() { +static lean_object* _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__2() { _start: { lean_object* x_1; @@ -12146,17 +12292,17 @@ x_1 = lean_mk_string_unchecked("maxRecDepth", 11, 11); return x_1; } } -static lean_object* _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__3() { +static lean_object* _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__1; -x_2 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__2; +x_1 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__1; +x_2 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__2; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__4() { +static lean_object* _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__4() { _start: { lean_object* x_1; lean_object* x_2; @@ -12166,32 +12312,32 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__5() { +static lean_object* _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__5() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__4; +x_1 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__4; x_2 = l_Lean_MessageData_ofFormat(x_1); return x_2; } } -static lean_object* _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__6() { +static lean_object* _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__3; -x_2 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__5; +x_1 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__3; +x_2 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__5; x_3 = lean_alloc_ctor(8, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_5 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__6; +x_5 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__6; x_6 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_6, 0, x_1); lean_ctor_set(x_6, 1, x_5); @@ -12201,7 +12347,7 @@ lean_ctor_set(x_7, 1, x_4); return x_7; } } -static lean_object* _init_l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___rarg___closed__1() { +static lean_object* _init_l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__5___rarg___closed__1() { _start: { lean_object* x_1; @@ -12209,38 +12355,38 @@ x_1 = l_Lean_Elab_unsupportedSyntaxExceptionId; return x_1; } } -static lean_object* _init_l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___rarg___closed__2() { +static lean_object* _init_l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__5___rarg___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___rarg___closed__1; +x_2 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__5___rarg___closed__1; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___rarg(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__5___rarg(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___rarg___closed__2; +x_2 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__5___rarg___closed__2; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__5(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___rarg), 1, 0); +x_3 = lean_alloc_closure((void*)(l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__5___rarg), 1, 0); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; @@ -12409,7 +12555,7 @@ return x_41; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__1___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { uint8_t x_5; lean_object* x_6; lean_object* x_7; @@ -12421,7 +12567,7 @@ lean_ctor_set(x_7, 1, x_4); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__1___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; lean_object* x_8; @@ -12432,7 +12578,7 @@ lean_ctor_set(x_8, 1, x_6); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__1___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; lean_object* x_8; @@ -12443,7 +12589,7 @@ lean_ctor_set(x_8, 1, x_6); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; @@ -12475,23 +12621,23 @@ x_16 = lean_ctor_get(x_14, 3); lean_inc(x_16); lean_dec(x_14); lean_inc(x_8); -x_17 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__1___boxed), 4, 1); +x_17 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__1___lambda__1___boxed), 4, 1); lean_closure_set(x_17, 0, x_8); lean_inc(x_12); x_18 = lean_alloc_closure((void*)(l_ReaderT_pure___at_Lean_Elab_liftMacroM___spec__2___rarg___boxed), 3, 1); lean_closure_set(x_18, 0, x_12); lean_inc(x_8); -x_19 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__2___boxed), 4, 1); +x_19 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__1___lambda__2___boxed), 4, 1); lean_closure_set(x_19, 0, x_8); lean_inc(x_16); lean_inc(x_12); lean_inc(x_8); -x_20 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__3___boxed), 6, 3); +x_20 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__1___lambda__3___boxed), 6, 3); lean_closure_set(x_20, 0, x_8); lean_closure_set(x_20, 1, x_12); lean_closure_set(x_20, 2, x_16); lean_inc(x_8); -x_21 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__4___boxed), 6, 3); +x_21 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__1___lambda__4___boxed), 6, 3); lean_closure_set(x_21, 0, x_8); lean_closure_set(x_21, 1, x_12); lean_closure_set(x_21, 2, x_16); @@ -12679,7 +12825,7 @@ lean_object* x_81; lean_object* x_82; lean_object* x_83; x_81 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_81, 0, x_78); x_82 = l_Lean_MessageData_ofFormat(x_81); -x_83 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__2(x_77, x_82, x_2, x_3, x_37); +x_83 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__2(x_77, x_82, x_2, x_3, x_37); lean_dec(x_77); return x_83; } @@ -12687,7 +12833,7 @@ else { lean_object* x_84; lean_dec(x_78); -x_84 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4(x_77, x_2, x_3, x_37); +x_84 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4(x_77, x_2, x_3, x_37); lean_dec(x_2); return x_84; } @@ -12696,7 +12842,7 @@ else { lean_object* x_85; lean_dec(x_2); -x_85 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___rarg(x_37); +x_85 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__5___rarg(x_37); return x_85; } } @@ -12833,7 +12979,7 @@ lean_object* x_122; lean_object* x_123; lean_object* x_124; x_122 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_122, 0, x_119); x_123 = l_Lean_MessageData_ofFormat(x_122); -x_124 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__2(x_118, x_123, x_2, x_3, x_87); +x_124 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__2(x_118, x_123, x_2, x_3, x_87); lean_dec(x_118); return x_124; } @@ -12841,7 +12987,7 @@ else { lean_object* x_125; lean_dec(x_119); -x_125 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4(x_118, x_2, x_3, x_87); +x_125 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4(x_118, x_2, x_3, x_87); lean_dec(x_2); return x_125; } @@ -12850,14 +12996,14 @@ else { lean_object* x_126; lean_dec(x_2); -x_126 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___rarg(x_87); +x_126 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__5___rarg(x_87); return x_126; } } } } } -LEAN_EXPORT lean_object* l_Lean_ScopedEnvExtension_add___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__6(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_ScopedEnvExtension_add___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__6(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; @@ -12878,7 +13024,7 @@ x_14 = lean_ctor_get(x_11, 0); x_15 = lean_ctor_get(x_11, 4); lean_dec(x_15); x_16 = l_Lean_ScopedEnvExtension_addCore___rarg(x_14, x_1, x_2, x_3, x_9); -x_17 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__2; +x_17 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__2; lean_ctor_set(x_11, 4, x_17); lean_ctor_set(x_11, 0, x_16); x_18 = lean_st_ref_set(x_7, x_11, x_12); @@ -12897,7 +13043,7 @@ if (x_23 == 0) lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; x_24 = lean_ctor_get(x_21, 1); lean_dec(x_24); -x_25 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5; +x_25 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5; lean_ctor_set(x_21, 1, x_25); x_26 = lean_st_ref_set(x_5, x_21, x_22); x_27 = !lean_is_exclusive(x_26); @@ -12935,7 +13081,7 @@ lean_inc(x_35); lean_inc(x_34); lean_inc(x_33); lean_dec(x_21); -x_37 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5; +x_37 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5; x_38 = lean_alloc_ctor(0, 5, 0); lean_ctor_set(x_38, 0, x_33); lean_ctor_set(x_38, 1, x_37); @@ -12981,7 +13127,7 @@ lean_inc(x_45); lean_inc(x_44); lean_dec(x_11); x_50 = l_Lean_ScopedEnvExtension_addCore___rarg(x_44, x_1, x_2, x_3, x_9); -x_51 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__2; +x_51 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__2; x_52 = lean_alloc_ctor(0, 7, 0); lean_ctor_set(x_52, 0, x_50); lean_ctor_set(x_52, 1, x_45); @@ -13019,7 +13165,7 @@ if (lean_is_exclusive(x_56)) { lean_dec_ref(x_56); x_62 = lean_box(0); } -x_63 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5; +x_63 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5; if (lean_is_scalar(x_62)) { x_64 = lean_alloc_ctor(0, 5, 0); } else { @@ -13053,7 +13199,7 @@ return x_69; } } } -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { uint8_t x_8; @@ -13122,7 +13268,7 @@ return x_28; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__8___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__8___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; lean_object* x_8; @@ -13133,7 +13279,7 @@ lean_ctor_set(x_8, 1, x_6); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; @@ -13193,7 +13339,7 @@ if (x_24 == 0) { lean_object* x_25; lean_object* x_26; x_25 = lean_box(0); -x_26 = l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__8___lambda__1(x_1, x_2, x_25, x_3, x_4, x_5); +x_26 = l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__8___lambda__1(x_1, x_2, x_25, x_3, x_4, x_5); return x_26; } else @@ -13232,7 +13378,7 @@ return x_36; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_5; @@ -13244,7 +13390,7 @@ lean_ctor_set(x_5, 1, x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; lean_object* x_6; @@ -13256,7 +13402,7 @@ lean_ctor_set(x_6, 1, x_3); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__3___closed__1() { _start: { lean_object* x_1; @@ -13264,17 +13410,17 @@ x_1 = lean_mk_string_unchecked("prioDefault", 11, 11); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__3___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__1; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__3___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__3___closed__3() { _start: { lean_object* x_1; @@ -13282,16 +13428,16 @@ x_1 = lean_mk_string_unchecked("default", 7, 7); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__3; +x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__3___closed__3; lean_inc(x_1); x_5 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_5, 0, x_1); lean_ctor_set(x_5, 1, x_4); -x_6 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__2; +x_6 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__3___closed__2; x_7 = l_Lean_Syntax_node1(x_1, x_6, x_5); x_8 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_8, 0, x_7); @@ -13299,7 +13445,7 @@ lean_ctor_set(x_8, 1, x_3); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { if (lean_obj_tag(x_1) == 0) @@ -13320,7 +13466,7 @@ return x_7; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; @@ -13382,7 +13528,7 @@ return x_24; } } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__1() { _start: { lean_object* x_1; @@ -13390,67 +13536,67 @@ x_1 = lean_alloc_closure((void*)(l_ReaderT_read___at_Lean_Macro_instMonadRefMacr return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__2() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__1___boxed), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__1___boxed), 3, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__1; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__2; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__1; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__2; x_3 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Macro_instMonadRefMacroM___spec__2___rarg), 4, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__4() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__2___boxed), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__2___boxed), 3, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__3; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__4; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__3; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__4; x_3 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Macro_instMonadRefMacroM___spec__2___rarg), 4, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__6() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__6() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___boxed), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__3___boxed), 3, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__7() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__5; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__6; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__5; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__6; x_3 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Macro_instMonadRefMacroM___spec__2___rarg), 4, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, uint8_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, uint8_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; @@ -13491,134 +13637,135 @@ lean_inc(x_9); x_26 = l_Lean_Meta_DiscrTree_mkPath(x_1, x_24, x_25, x_23, x_9, x_10, x_11, 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; 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_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; lean_object* x_34; x_27 = lean_ctor_get(x_26, 0); lean_inc(x_27); x_28 = lean_ctor_get(x_26, 1); lean_inc(x_28); lean_dec(x_26); -x_29 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__4), 4, 1); +x_29 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__4), 4, 1); lean_closure_set(x_29, 0, x_2); -x_30 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__7; +x_30 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__7; x_31 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Macro_instMonadRefMacroM___spec__2___rarg), 4, 2); lean_closure_set(x_31, 0, x_30); lean_closure_set(x_31, 1, x_29); -x_32 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___boxed), 4, 1); +x_32 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__1___boxed), 4, 1); lean_closure_set(x_32, 0, x_31); -x_33 = l_Lean_liftCommandElabM___rarg(x_32, x_10, x_11, x_28); -if (lean_obj_tag(x_33) == 0) +x_33 = 1; +x_34 = l_Lean_liftCommandElabM___rarg(x_32, x_33, x_10, x_11, x_28); +if (lean_obj_tag(x_34) == 0) { -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_34 = lean_ctor_get(x_33, 0); -lean_inc(x_34); -x_35 = lean_ctor_get(x_33, 1); +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_35 = lean_ctor_get(x_34, 0); lean_inc(x_35); -lean_dec(x_33); +x_36 = lean_ctor_get(x_34, 1); +lean_inc(x_36); +lean_dec(x_34); lean_inc(x_3); -x_36 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_36, 0, x_3); -lean_ctor_set(x_36, 1, x_34); -lean_ctor_set(x_36, 2, x_27); -x_37 = l_Lean_Elab_Tactic_Ext_getExtTheorems___closed__1; +x_37 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_37, 0, x_3); +lean_ctor_set(x_37, 1, x_35); +lean_ctor_set(x_37, 2, x_27); +x_38 = l_Lean_Elab_Tactic_Ext_getExtTheorems___closed__1; lean_inc(x_10); -x_38 = l_Lean_ScopedEnvExtension_add___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__6(x_37, x_36, x_4, x_8, x_9, x_10, x_11, x_35); +x_39 = l_Lean_ScopedEnvExtension_add___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__6(x_38, x_37, x_4, x_8, x_9, x_10, x_11, x_36); lean_dec(x_9); lean_dec(x_8); if (x_5 == 0) { -uint8_t x_39; +uint8_t x_40; lean_dec(x_11); lean_dec(x_10); lean_dec(x_6); lean_dec(x_3); -x_39 = !lean_is_exclusive(x_38); -if (x_39 == 0) +x_40 = !lean_is_exclusive(x_39); +if (x_40 == 0) { -lean_object* x_40; lean_object* x_41; -x_40 = lean_ctor_get(x_38, 0); -lean_dec(x_40); -x_41 = lean_box(0); -lean_ctor_set(x_38, 0, x_41); -return x_38; +lean_object* x_41; lean_object* x_42; +x_41 = lean_ctor_get(x_39, 0); +lean_dec(x_41); +x_42 = lean_box(0); +lean_ctor_set(x_39, 0, x_42); +return x_39; } else { -lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_ctor_get(x_38, 1); -lean_inc(x_42); -lean_dec(x_38); -x_43 = lean_box(0); -x_44 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_44, 0, x_43); -lean_ctor_set(x_44, 1, x_42); -return x_44; +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_39, 1); +lean_inc(x_43); +lean_dec(x_39); +x_44 = lean_box(0); +x_45 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_45, 0, x_44); +lean_ctor_set(x_45, 1, x_43); +return x_45; } } else { -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_38, 1); -lean_inc(x_45); -lean_dec(x_38); -x_46 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__5___boxed), 5, 2); -lean_closure_set(x_46, 0, x_6); -lean_closure_set(x_46, 1, x_3); -x_47 = l_Lean_liftCommandElabM___rarg(x_46, x_10, x_11, x_45); +lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_46 = lean_ctor_get(x_39, 1); +lean_inc(x_46); +lean_dec(x_39); +x_47 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__5___boxed), 5, 2); +lean_closure_set(x_47, 0, x_6); +lean_closure_set(x_47, 1, x_3); +x_48 = l_Lean_liftCommandElabM___rarg(x_47, x_33, x_10, x_11, x_46); lean_dec(x_11); lean_dec(x_10); -if (lean_obj_tag(x_47) == 0) +if (lean_obj_tag(x_48) == 0) { -uint8_t x_48; -x_48 = !lean_is_exclusive(x_47); -if (x_48 == 0) +uint8_t x_49; +x_49 = !lean_is_exclusive(x_48); +if (x_49 == 0) { -lean_object* x_49; lean_object* x_50; -x_49 = lean_ctor_get(x_47, 0); -lean_dec(x_49); -x_50 = lean_box(0); -lean_ctor_set(x_47, 0, x_50); -return x_47; +lean_object* x_50; lean_object* x_51; +x_50 = lean_ctor_get(x_48, 0); +lean_dec(x_50); +x_51 = lean_box(0); +lean_ctor_set(x_48, 0, x_51); +return x_48; } else { -lean_object* x_51; lean_object* x_52; lean_object* x_53; -x_51 = lean_ctor_get(x_47, 1); -lean_inc(x_51); -lean_dec(x_47); -x_52 = lean_box(0); -x_53 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_53, 0, x_52); -lean_ctor_set(x_53, 1, x_51); -return x_53; +lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_52 = lean_ctor_get(x_48, 1); +lean_inc(x_52); +lean_dec(x_48); +x_53 = lean_box(0); +x_54 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_54, 0, x_53); +lean_ctor_set(x_54, 1, x_52); +return x_54; } } else { -uint8_t x_54; -x_54 = !lean_is_exclusive(x_47); -if (x_54 == 0) +uint8_t x_55; +x_55 = !lean_is_exclusive(x_48); +if (x_55 == 0) { -return x_47; +return x_48; } else { -lean_object* x_55; lean_object* x_56; lean_object* x_57; -x_55 = lean_ctor_get(x_47, 0); -x_56 = lean_ctor_get(x_47, 1); +lean_object* x_56; lean_object* x_57; lean_object* x_58; +x_56 = lean_ctor_get(x_48, 0); +x_57 = lean_ctor_get(x_48, 1); +lean_inc(x_57); lean_inc(x_56); -lean_inc(x_55); -lean_dec(x_47); -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_48); +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; +uint8_t x_59; lean_dec(x_27); lean_dec(x_11); lean_dec(x_10); @@ -13626,29 +13773,29 @@ lean_dec(x_9); lean_dec(x_8); lean_dec(x_6); lean_dec(x_3); -x_58 = !lean_is_exclusive(x_33); -if (x_58 == 0) +x_59 = !lean_is_exclusive(x_34); +if (x_59 == 0) { -return x_33; +return x_34; } else { -lean_object* x_59; lean_object* x_60; lean_object* x_61; -x_59 = lean_ctor_get(x_33, 0); -x_60 = lean_ctor_get(x_33, 1); +lean_object* x_60; lean_object* x_61; lean_object* x_62; +x_60 = lean_ctor_get(x_34, 0); +x_61 = lean_ctor_get(x_34, 1); +lean_inc(x_61); lean_inc(x_60); -lean_inc(x_59); -lean_dec(x_33); -x_61 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_61, 0, x_59); -lean_ctor_set(x_61, 1, x_60); -return x_61; +lean_dec(x_34); +x_62 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_62, 0, x_60); +lean_ctor_set(x_62, 1, x_61); +return x_62; } } } else { -uint8_t x_62; +uint8_t x_63; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -13656,232 +13803,233 @@ lean_dec(x_8); lean_dec(x_6); lean_dec(x_3); lean_dec(x_2); -x_62 = !lean_is_exclusive(x_26); -if (x_62 == 0) +x_63 = !lean_is_exclusive(x_26); +if (x_63 == 0) { return x_26; } else { -lean_object* x_63; lean_object* x_64; lean_object* x_65; -x_63 = lean_ctor_get(x_26, 0); -x_64 = lean_ctor_get(x_26, 1); +lean_object* x_64; lean_object* x_65; lean_object* x_66; +x_64 = lean_ctor_get(x_26, 0); +x_65 = lean_ctor_get(x_26, 1); +lean_inc(x_65); lean_inc(x_64); -lean_inc(x_63); lean_dec(x_26); -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; +x_66 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_66, 0, x_64); +lean_ctor_set(x_66, 1, x_65); +return x_66; } } } else { -uint8_t x_66; uint8_t x_67; uint8_t x_68; uint8_t x_69; uint8_t x_70; uint8_t x_71; uint8_t x_72; uint8_t x_73; uint8_t 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; lean_object* x_81; lean_object* x_82; lean_object* x_83; uint8_t x_84; lean_object* x_85; -x_66 = lean_ctor_get_uint8(x_8, sizeof(void*)*6); -x_67 = lean_ctor_get_uint8(x_8, sizeof(void*)*6 + 1); -x_68 = lean_ctor_get_uint8(x_13, 0); -x_69 = lean_ctor_get_uint8(x_13, 1); -x_70 = lean_ctor_get_uint8(x_13, 2); -x_71 = lean_ctor_get_uint8(x_13, 3); -x_72 = lean_ctor_get_uint8(x_13, 4); -x_73 = lean_ctor_get_uint8(x_13, 5); -x_74 = lean_ctor_get_uint8(x_13, 6); -x_75 = lean_ctor_get_uint8(x_13, 7); -x_76 = lean_ctor_get_uint8(x_13, 8); -x_77 = lean_ctor_get_uint8(x_13, 10); -x_78 = lean_ctor_get_uint8(x_13, 11); -x_79 = lean_ctor_get_uint8(x_13, 12); +uint8_t x_67; uint8_t x_68; uint8_t x_69; uint8_t x_70; uint8_t x_71; uint8_t x_72; uint8_t x_73; uint8_t 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; lean_object* x_82; lean_object* x_83; lean_object* x_84; uint8_t x_85; lean_object* x_86; +x_67 = lean_ctor_get_uint8(x_8, sizeof(void*)*6); +x_68 = lean_ctor_get_uint8(x_8, sizeof(void*)*6 + 1); +x_69 = lean_ctor_get_uint8(x_13, 0); +x_70 = lean_ctor_get_uint8(x_13, 1); +x_71 = lean_ctor_get_uint8(x_13, 2); +x_72 = lean_ctor_get_uint8(x_13, 3); +x_73 = lean_ctor_get_uint8(x_13, 4); +x_74 = lean_ctor_get_uint8(x_13, 5); +x_75 = lean_ctor_get_uint8(x_13, 6); +x_76 = lean_ctor_get_uint8(x_13, 7); +x_77 = lean_ctor_get_uint8(x_13, 8); +x_78 = lean_ctor_get_uint8(x_13, 10); +x_79 = lean_ctor_get_uint8(x_13, 11); +x_80 = lean_ctor_get_uint8(x_13, 12); lean_dec(x_13); -x_80 = 2; -x_81 = lean_alloc_ctor(0, 0, 13); -lean_ctor_set_uint8(x_81, 0, x_68); -lean_ctor_set_uint8(x_81, 1, x_69); -lean_ctor_set_uint8(x_81, 2, x_70); -lean_ctor_set_uint8(x_81, 3, x_71); -lean_ctor_set_uint8(x_81, 4, x_72); -lean_ctor_set_uint8(x_81, 5, x_73); -lean_ctor_set_uint8(x_81, 6, x_74); -lean_ctor_set_uint8(x_81, 7, x_75); -lean_ctor_set_uint8(x_81, 8, x_76); -lean_ctor_set_uint8(x_81, 9, x_80); -lean_ctor_set_uint8(x_81, 10, x_77); -lean_ctor_set_uint8(x_81, 11, x_78); -lean_ctor_set_uint8(x_81, 12, x_79); -x_82 = lean_alloc_ctor(0, 6, 2); -lean_ctor_set(x_82, 0, x_81); -lean_ctor_set(x_82, 1, x_14); -lean_ctor_set(x_82, 2, x_15); -lean_ctor_set(x_82, 3, x_16); -lean_ctor_set(x_82, 4, x_17); -lean_ctor_set(x_82, 5, x_18); -lean_ctor_set_uint8(x_82, sizeof(void*)*6, x_66); -lean_ctor_set_uint8(x_82, sizeof(void*)*6 + 1, x_67); -x_83 = l_Lean_Elab_Tactic_Ext_extExt_config; -x_84 = 0; +x_81 = 2; +x_82 = lean_alloc_ctor(0, 0, 13); +lean_ctor_set_uint8(x_82, 0, x_69); +lean_ctor_set_uint8(x_82, 1, x_70); +lean_ctor_set_uint8(x_82, 2, x_71); +lean_ctor_set_uint8(x_82, 3, x_72); +lean_ctor_set_uint8(x_82, 4, x_73); +lean_ctor_set_uint8(x_82, 5, x_74); +lean_ctor_set_uint8(x_82, 6, x_75); +lean_ctor_set_uint8(x_82, 7, x_76); +lean_ctor_set_uint8(x_82, 8, x_77); +lean_ctor_set_uint8(x_82, 9, x_81); +lean_ctor_set_uint8(x_82, 10, x_78); +lean_ctor_set_uint8(x_82, 11, x_79); +lean_ctor_set_uint8(x_82, 12, x_80); +x_83 = lean_alloc_ctor(0, 6, 2); +lean_ctor_set(x_83, 0, x_82); +lean_ctor_set(x_83, 1, x_14); +lean_ctor_set(x_83, 2, x_15); +lean_ctor_set(x_83, 3, x_16); +lean_ctor_set(x_83, 4, x_17); +lean_ctor_set(x_83, 5, x_18); +lean_ctor_set_uint8(x_83, sizeof(void*)*6, x_67); +lean_ctor_set_uint8(x_83, sizeof(void*)*6 + 1, x_68); +x_84 = l_Lean_Elab_Tactic_Ext_extExt_config; +x_85 = 0; lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -x_85 = l_Lean_Meta_DiscrTree_mkPath(x_1, x_83, x_84, x_82, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_85) == 0) +x_86 = l_Lean_Meta_DiscrTree_mkPath(x_1, x_84, x_85, x_83, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_86) == 0) { -lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; -x_86 = lean_ctor_get(x_85, 0); -lean_inc(x_86); -x_87 = lean_ctor_get(x_85, 1); +lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; uint8_t x_93; lean_object* x_94; +x_87 = lean_ctor_get(x_86, 0); lean_inc(x_87); -lean_dec(x_85); -x_88 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__4), 4, 1); -lean_closure_set(x_88, 0, x_2); -x_89 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__7; -x_90 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Macro_instMonadRefMacroM___spec__2___rarg), 4, 2); -lean_closure_set(x_90, 0, x_89); -lean_closure_set(x_90, 1, x_88); -x_91 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___boxed), 4, 1); +x_88 = lean_ctor_get(x_86, 1); +lean_inc(x_88); +lean_dec(x_86); +x_89 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__4), 4, 1); +lean_closure_set(x_89, 0, x_2); +x_90 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__7; +x_91 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Macro_instMonadRefMacroM___spec__2___rarg), 4, 2); lean_closure_set(x_91, 0, x_90); -x_92 = l_Lean_liftCommandElabM___rarg(x_91, x_10, x_11, x_87); -if (lean_obj_tag(x_92) == 0) -{ -lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; -x_93 = lean_ctor_get(x_92, 0); -lean_inc(x_93); -x_94 = lean_ctor_get(x_92, 1); -lean_inc(x_94); -lean_dec(x_92); +lean_closure_set(x_91, 1, x_89); +x_92 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__1___boxed), 4, 1); +lean_closure_set(x_92, 0, x_91); +x_93 = 1; +x_94 = l_Lean_liftCommandElabM___rarg(x_92, x_93, x_10, x_11, x_88); +if (lean_obj_tag(x_94) == 0) +{ +lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; +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_3); -x_95 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_95, 0, x_3); -lean_ctor_set(x_95, 1, x_93); -lean_ctor_set(x_95, 2, x_86); -x_96 = l_Lean_Elab_Tactic_Ext_getExtTheorems___closed__1; +x_97 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_97, 0, x_3); +lean_ctor_set(x_97, 1, x_95); +lean_ctor_set(x_97, 2, x_87); +x_98 = l_Lean_Elab_Tactic_Ext_getExtTheorems___closed__1; lean_inc(x_10); -x_97 = l_Lean_ScopedEnvExtension_add___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__6(x_96, x_95, x_4, x_8, x_9, x_10, x_11, x_94); +x_99 = l_Lean_ScopedEnvExtension_add___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__6(x_98, x_97, x_4, x_8, x_9, x_10, x_11, x_96); lean_dec(x_9); lean_dec(x_8); if (x_5 == 0) { -lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; +lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_dec(x_11); lean_dec(x_10); lean_dec(x_6); lean_dec(x_3); -x_98 = lean_ctor_get(x_97, 1); -lean_inc(x_98); -if (lean_is_exclusive(x_97)) { - lean_ctor_release(x_97, 0); - lean_ctor_release(x_97, 1); - x_99 = x_97; +x_100 = lean_ctor_get(x_99, 1); +lean_inc(x_100); +if (lean_is_exclusive(x_99)) { + lean_ctor_release(x_99, 0); + lean_ctor_release(x_99, 1); + x_101 = x_99; } else { - lean_dec_ref(x_97); - x_99 = lean_box(0); + lean_dec_ref(x_99); + x_101 = lean_box(0); } -x_100 = lean_box(0); -if (lean_is_scalar(x_99)) { - x_101 = lean_alloc_ctor(0, 2, 0); +x_102 = lean_box(0); +if (lean_is_scalar(x_101)) { + x_103 = lean_alloc_ctor(0, 2, 0); } else { - x_101 = x_99; + x_103 = x_101; } -lean_ctor_set(x_101, 0, x_100); -lean_ctor_set(x_101, 1, x_98); -return x_101; +lean_ctor_set(x_103, 0, x_102); +lean_ctor_set(x_103, 1, x_100); +return x_103; } else { -lean_object* x_102; lean_object* x_103; lean_object* x_104; -x_102 = lean_ctor_get(x_97, 1); -lean_inc(x_102); -lean_dec(x_97); -x_103 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__5___boxed), 5, 2); -lean_closure_set(x_103, 0, x_6); -lean_closure_set(x_103, 1, x_3); -x_104 = l_Lean_liftCommandElabM___rarg(x_103, x_10, x_11, x_102); +lean_object* x_104; lean_object* x_105; lean_object* x_106; +x_104 = lean_ctor_get(x_99, 1); +lean_inc(x_104); +lean_dec(x_99); +x_105 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__5___boxed), 5, 2); +lean_closure_set(x_105, 0, x_6); +lean_closure_set(x_105, 1, x_3); +x_106 = l_Lean_liftCommandElabM___rarg(x_105, x_93, x_10, x_11, x_104); lean_dec(x_11); lean_dec(x_10); -if (lean_obj_tag(x_104) == 0) -{ -lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; -x_105 = lean_ctor_get(x_104, 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; +if (lean_obj_tag(x_106) == 0) +{ +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); +if (lean_is_exclusive(x_106)) { + lean_ctor_release(x_106, 0); + lean_ctor_release(x_106, 1); + x_108 = x_106; } else { - lean_dec_ref(x_104); - x_106 = lean_box(0); + lean_dec_ref(x_106); + x_108 = lean_box(0); } -x_107 = lean_box(0); -if (lean_is_scalar(x_106)) { - x_108 = lean_alloc_ctor(0, 2, 0); +x_109 = lean_box(0); +if (lean_is_scalar(x_108)) { + x_110 = lean_alloc_ctor(0, 2, 0); } else { - x_108 = x_106; + x_110 = x_108; } -lean_ctor_set(x_108, 0, x_107); -lean_ctor_set(x_108, 1, x_105); -return x_108; +lean_ctor_set(x_110, 0, x_109); +lean_ctor_set(x_110, 1, x_107); +return x_110; } else { -lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; -x_109 = lean_ctor_get(x_104, 0); -lean_inc(x_109); -x_110 = lean_ctor_get(x_104, 1); -lean_inc(x_110); -if (lean_is_exclusive(x_104)) { - lean_ctor_release(x_104, 0); - lean_ctor_release(x_104, 1); - x_111 = x_104; +lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; +x_111 = lean_ctor_get(x_106, 0); +lean_inc(x_111); +x_112 = lean_ctor_get(x_106, 1); +lean_inc(x_112); +if (lean_is_exclusive(x_106)) { + lean_ctor_release(x_106, 0); + lean_ctor_release(x_106, 1); + x_113 = x_106; } else { - lean_dec_ref(x_104); - x_111 = lean_box(0); + lean_dec_ref(x_106); + x_113 = lean_box(0); } -if (lean_is_scalar(x_111)) { - x_112 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_113)) { + x_114 = lean_alloc_ctor(1, 2, 0); } else { - x_112 = x_111; + x_114 = x_113; } -lean_ctor_set(x_112, 0, x_109); -lean_ctor_set(x_112, 1, x_110); -return x_112; +lean_ctor_set(x_114, 0, x_111); +lean_ctor_set(x_114, 1, x_112); +return x_114; } } } else { -lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; -lean_dec(x_86); +lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; +lean_dec(x_87); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_6); lean_dec(x_3); -x_113 = lean_ctor_get(x_92, 0); -lean_inc(x_113); -x_114 = lean_ctor_get(x_92, 1); -lean_inc(x_114); -if (lean_is_exclusive(x_92)) { - lean_ctor_release(x_92, 0); - lean_ctor_release(x_92, 1); - x_115 = x_92; +x_115 = lean_ctor_get(x_94, 0); +lean_inc(x_115); +x_116 = lean_ctor_get(x_94, 1); +lean_inc(x_116); +if (lean_is_exclusive(x_94)) { + lean_ctor_release(x_94, 0); + lean_ctor_release(x_94, 1); + x_117 = x_94; } else { - lean_dec_ref(x_92); - x_115 = lean_box(0); + lean_dec_ref(x_94); + x_117 = lean_box(0); } -if (lean_is_scalar(x_115)) { - x_116 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_117)) { + x_118 = lean_alloc_ctor(1, 2, 0); } else { - x_116 = x_115; + x_118 = x_117; } -lean_ctor_set(x_116, 0, x_113); -lean_ctor_set(x_116, 1, x_114); -return x_116; +lean_ctor_set(x_118, 0, x_115); +lean_ctor_set(x_118, 1, x_116); +return x_118; } } else { -lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; +lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -13889,31 +14037,31 @@ lean_dec(x_8); lean_dec(x_6); lean_dec(x_3); lean_dec(x_2); -x_117 = lean_ctor_get(x_85, 0); -lean_inc(x_117); -x_118 = lean_ctor_get(x_85, 1); -lean_inc(x_118); -if (lean_is_exclusive(x_85)) { - lean_ctor_release(x_85, 0); - lean_ctor_release(x_85, 1); - x_119 = x_85; +x_119 = lean_ctor_get(x_86, 0); +lean_inc(x_119); +x_120 = lean_ctor_get(x_86, 1); +lean_inc(x_120); +if (lean_is_exclusive(x_86)) { + lean_ctor_release(x_86, 0); + lean_ctor_release(x_86, 1); + x_121 = x_86; } else { - lean_dec_ref(x_85); - x_119 = lean_box(0); + lean_dec_ref(x_86); + x_121 = lean_box(0); } -if (lean_is_scalar(x_119)) { - x_120 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_121)) { + x_122 = lean_alloc_ctor(1, 2, 0); } else { - x_120 = x_119; + x_122 = x_121; } -lean_ctor_set(x_120, 0, x_117); -lean_ctor_set(x_120, 1, x_118); -return x_120; +lean_ctor_set(x_122, 0, x_119); +lean_ctor_set(x_122, 1, x_120); +return x_122; } } } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__7___closed__1() { _start: { lean_object* x_1; @@ -13921,16 +14069,16 @@ x_1 = lean_mk_string_unchecked("@[ext] attribute only applies to structures and return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__7___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7___closed__1; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__7___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__7(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; @@ -14006,7 +14154,7 @@ lean_dec(x_38); lean_inc(x_37); x_39 = l_Lean_MessageData_ofExpr(x_37); x_40 = l_Lean_indentD(x_39); -x_41 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7___closed__2; +x_41 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__7___closed__2; lean_ctor_set_tag(x_33, 7); lean_ctor_set(x_33, 1, x_40); lean_ctor_set(x_33, 0, x_41); @@ -14117,7 +14265,7 @@ else lean_object* x_64; lean_object* x_65; lean_dec(x_31); x_64 = lean_box(0); -x_65 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6(x_49, x_2, x_6, x_3, x_4, x_5, x_64, x_8, x_9, x_10, x_11, x_35); +x_65 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6(x_49, x_2, x_6, x_3, x_4, x_5, x_64, x_8, x_9, x_10, x_11, x_35); return x_65; } } @@ -14132,7 +14280,7 @@ lean_dec(x_33); lean_inc(x_66); x_67 = l_Lean_MessageData_ofExpr(x_66); x_68 = l_Lean_indentD(x_67); -x_69 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7___closed__2; +x_69 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__7___closed__2; x_70 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_70, 0, x_69); lean_ctor_set(x_70, 1, x_68); @@ -14247,7 +14395,7 @@ else lean_object* x_93; lean_object* x_94; lean_dec(x_31); x_93 = lean_box(0); -x_94 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6(x_78, x_2, x_6, x_3, x_4, x_5, x_93, x_8, x_9, x_10, x_11, x_35); +x_94 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6(x_78, x_2, x_6, x_3, x_4, x_5, x_93, x_8, x_9, x_10, x_11, x_35); return x_94; } } @@ -14276,7 +14424,7 @@ if (lean_is_exclusive(x_95)) { lean_inc(x_97); x_99 = l_Lean_MessageData_ofExpr(x_97); x_100 = l_Lean_indentD(x_99); -x_101 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7___closed__2; +x_101 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__7___closed__2; if (lean_is_scalar(x_98)) { x_102 = lean_alloc_ctor(7, 2, 0); } else { @@ -14396,7 +14544,7 @@ else lean_object* x_126; lean_object* x_127; lean_dec(x_104); x_126 = lean_box(0); -x_127 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6(x_111, x_2, x_6, x_3, x_4, x_5, x_126, x_8, x_9, x_10, x_11, x_96); +x_127 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6(x_111, x_2, x_6, x_3, x_4, x_5, x_126, x_8, x_9, x_10, x_11, x_96); return x_127; } } @@ -14512,7 +14660,7 @@ if (lean_is_exclusive(x_153)) { lean_inc(x_156); x_158 = l_Lean_MessageData_ofExpr(x_156); x_159 = l_Lean_indentD(x_158); -x_160 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7___closed__2; +x_160 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__7___closed__2; if (lean_is_scalar(x_157)) { x_161 = lean_alloc_ctor(7, 2, 0); } else { @@ -14637,7 +14785,7 @@ else lean_object* x_185; lean_object* x_186; lean_dec(x_163); x_185 = lean_box(0); -x_186 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6(x_170, x_2, x_6, x_3, x_4, x_5, x_185, x_8, x_9, x_10, x_11, x_155); +x_186 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6(x_170, x_2, x_6, x_3, x_4, x_5, x_185, x_8, x_9, x_10, x_11, x_155); return x_186; } } @@ -14707,7 +14855,7 @@ return x_194; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__8(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__8(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; @@ -14769,7 +14917,7 @@ return x_25; } } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__9___closed__1() { _start: { lean_object* x_1; @@ -14777,16 +14925,16 @@ x_1 = lean_mk_string_unchecked("unexpected 'flat' configuration on @[ext] theore return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__9___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9___closed__1; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__9___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__9(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; @@ -14799,64 +14947,64 @@ if (lean_obj_tag(x_15) == 0) { lean_inc(x_2); x_17 = x_2; -goto block_50; +goto block_51; } else { -uint8_t x_51; -x_51 = !lean_is_exclusive(x_15); -if (x_51 == 0) +uint8_t x_52; +x_52 = !lean_is_exclusive(x_15); +if (x_52 == 0) { x_17 = x_15; -goto block_50; +goto block_51; } else { -lean_object* x_52; lean_object* x_53; -x_52 = lean_ctor_get(x_15, 0); -lean_inc(x_52); +lean_object* x_53; lean_object* x_54; +x_53 = lean_ctor_get(x_15, 0); +lean_inc(x_53); lean_dec(x_15); -x_53 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_53, 0, x_52); -x_17 = x_53; -goto block_50; +x_54 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_54, 0, x_53); +x_17 = x_54; +goto block_51; } } -block_50: +block_51: { uint8_t x_18; if (lean_obj_tag(x_5) == 0) { -uint8_t x_48; -x_48 = 1; -x_18 = x_48; -goto block_47; +uint8_t x_49; +x_49 = 1; +x_18 = x_49; +goto block_48; } else { -uint8_t x_49; -x_49 = 0; -x_18 = x_49; -goto block_47; +uint8_t x_50; +x_50 = 0; +x_18 = x_50; +goto block_48; } -block_47: +block_48: { uint8_t x_19; if (lean_obj_tag(x_7) == 0) { -uint8_t x_45; -x_45 = 1; -x_19 = x_45; -goto block_44; +uint8_t x_46; +x_46 = 1; +x_19 = x_46; +goto block_45; } else { -uint8_t x_46; -x_46 = 0; -x_19 = x_46; -goto block_44; +uint8_t x_47; +x_47 = 0; +x_19 = x_47; +goto block_45; } -block_44: +block_45: { lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; x_20 = lean_ctor_get(x_16, 0); @@ -14876,7 +15024,7 @@ if (lean_obj_tag(x_7) == 0) { lean_object* x_24; lean_object* x_25; x_24 = lean_box(0); -x_25 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7(x_2, x_17, x_3, x_18, x_1, x_4, x_24, x_8, x_9, x_10, x_11, x_21); +x_25 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__7(x_2, x_17, x_3, x_18, x_1, x_4, x_24, x_8, x_9, x_10, x_11, x_21); lean_dec(x_2); return x_25; } @@ -14888,8 +15036,8 @@ lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); x_26 = lean_ctor_get(x_7, 0); -x_27 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9___closed__2; -x_28 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__7(x_26, x_27, x_8, x_9, x_10, x_11, x_21); +x_27 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__9___closed__2; +x_28 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__7(x_26, x_27, x_8, x_9, x_10, x_11, x_21); lean_dec(x_11); lean_dec(x_9); lean_dec(x_8); @@ -14915,30 +15063,31 @@ return x_32; } else { -lean_object* x_33; lean_object* x_34; lean_object* x_35; +lean_object* x_33; lean_object* x_34; uint8_t x_35; lean_object* x_36; x_33 = lean_box(x_19); lean_inc(x_1); -x_34 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__8___boxed), 6, 3); +x_34 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__8___boxed), 6, 3); lean_closure_set(x_34, 0, x_1); lean_closure_set(x_34, 1, x_4); lean_closure_set(x_34, 2, x_33); -x_35 = l_Lean_liftCommandElabM___rarg(x_34, x_10, x_11, x_21); -if (lean_obj_tag(x_35) == 0) +x_35 = 1; +x_36 = l_Lean_liftCommandElabM___rarg(x_34, x_35, x_10, x_11, x_21); +if (lean_obj_tag(x_36) == 0) { -lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_36 = lean_ctor_get(x_35, 0); -lean_inc(x_36); -x_37 = lean_ctor_get(x_35, 1); +lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_37 = lean_ctor_get(x_36, 0); lean_inc(x_37); -lean_dec(x_35); -x_38 = lean_box(0); -x_39 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7(x_2, x_17, x_3, x_18, x_1, x_36, x_38, x_8, x_9, x_10, x_11, x_37); +x_38 = lean_ctor_get(x_36, 1); +lean_inc(x_38); +lean_dec(x_36); +x_39 = lean_box(0); +x_40 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__7(x_2, x_17, x_3, x_18, x_1, x_37, x_39, x_8, x_9, x_10, x_11, x_38); lean_dec(x_2); -return x_39; +return x_40; } else { -uint8_t x_40; +uint8_t x_41; lean_dec(x_17); lean_dec(x_11); lean_dec(x_10); @@ -14946,23 +15095,23 @@ lean_dec(x_9); lean_dec(x_8); lean_dec(x_2); lean_dec(x_1); -x_40 = !lean_is_exclusive(x_35); -if (x_40 == 0) +x_41 = !lean_is_exclusive(x_36); +if (x_41 == 0) { -return x_35; +return x_36; } else { -lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_ctor_get(x_35, 0); -x_42 = lean_ctor_get(x_35, 1); +lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_42 = lean_ctor_get(x_36, 0); +x_43 = lean_ctor_get(x_36, 1); +lean_inc(x_43); lean_inc(x_42); -lean_inc(x_41); -lean_dec(x_35); -x_43 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_43, 0, x_41); -lean_ctor_set(x_43, 1, x_42); -return x_43; +lean_dec(x_36); +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; } } } @@ -14971,7 +15120,7 @@ return x_43; } } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__1() { _start: { lean_object* x_1; @@ -14979,16 +15128,16 @@ x_1 = lean_mk_string_unchecked("invalid syntax for 'ext' attribute", 34, 34); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__1; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__3() { _start: { lean_object* x_1; @@ -14996,7 +15145,7 @@ x_1 = lean_mk_string_unchecked("Attr", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__4() { _start: { lean_object* x_1; @@ -15004,19 +15153,19 @@ x_1 = lean_mk_string_unchecked("extFlat", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__1; x_2 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__2; -x_3 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__3; -x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__4; +x_3 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__3; +x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__4; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { lean_object* x_12; lean_object* x_13; uint8_t x_14; @@ -15036,7 +15185,7 @@ lean_dec(x_13); lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_17 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__2; +x_17 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__2; x_18 = l_Lean_throwError___at_Lean_Meta_setInlineAttribute___spec__1(x_17, x_7, x_8, x_9, x_10, x_11); lean_dec(x_10); lean_dec(x_9); @@ -15050,7 +15199,7 @@ lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; x_19 = lean_unsigned_to_nat(0u); x_20 = l_Lean_Syntax_getArg(x_13, x_19); lean_dec(x_13); -x_21 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__5; +x_21 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__5; lean_inc(x_20); x_22 = l_Lean_Syntax_isOfKind(x_20, x_21); if (x_22 == 0) @@ -15060,7 +15209,7 @@ lean_dec(x_20); lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_23 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__2; +x_23 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__2; x_24 = l_Lean_throwError___at_Lean_Meta_setInlineAttribute___spec__1(x_23, x_7, x_8, x_9, x_10, x_11); lean_dec(x_10); lean_dec(x_9); @@ -15077,7 +15226,7 @@ lean_dec(x_20); x_27 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_27, 0, x_26); x_28 = lean_box(0); -x_29 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9(x_1, x_2, x_3, x_4, x_6, x_28, x_27, x_7, x_8, x_9, x_10, x_11); +x_29 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__9(x_1, x_2, x_3, x_4, x_6, x_28, x_27, x_7, x_8, x_9, x_10, x_11); lean_dec(x_27); return x_29; } @@ -15089,25 +15238,25 @@ lean_object* x_30; lean_object* x_31; lean_dec(x_13); x_30 = lean_box(0); lean_inc(x_2); -x_31 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9(x_1, x_2, x_3, x_4, x_6, x_30, x_2, x_7, x_8, x_9, x_10, x_11); +x_31 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__9(x_1, x_2, x_3, x_4, x_6, x_30, x_2, x_7, x_8, x_9, x_10, x_11); lean_dec(x_2); return x_31; } } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__1; x_2 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__2; -x_3 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__3; +x_3 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__3; x_4 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__5___closed__1; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__2() { _start: { uint8_t x_1; uint8_t x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; @@ -15132,12 +15281,12 @@ lean_ctor_set_uint8(x_5, 12, x_2); return x_5; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; uint8_t x_6; lean_object* x_7; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__2; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__2; x_3 = l_Lean_Elab_Tactic_Ext_mkExtType___closed__6; x_4 = l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___lambda__2___closed__1; x_5 = lean_unsigned_to_nat(0u); @@ -15154,7 +15303,7 @@ lean_ctor_set_uint8(x_7, sizeof(void*)*6 + 1, x_6); return x_7; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -15173,7 +15322,7 @@ lean_ctor_set(x_3, 8, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__5() { _start: { lean_object* x_1; lean_object* x_2; @@ -15186,15 +15335,15 @@ lean_ctor_set(x_2, 3, x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__6() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__4; -x_3 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__4; +x_3 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5; x_4 = l_Lean_Elab_Tactic_Ext_mkExtType___closed__5; -x_5 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__5; +x_5 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__5; x_6 = lean_alloc_ctor(0, 5, 0); lean_ctor_set(x_6, 0, x_2); lean_ctor_set(x_6, 1, x_3); @@ -15204,7 +15353,7 @@ lean_ctor_set(x_6, 4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__7() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__7() { _start: { lean_object* x_1; @@ -15212,27 +15361,27 @@ x_1 = lean_mk_string_unchecked("extIff", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__8() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__1; x_2 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__2; -x_3 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__3; -x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__7; +x_3 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__3; +x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__7; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; uint8_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; lean_object* x_13; lean_object* x_14; -x_7 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__1; +x_7 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__1; lean_inc(x_2); x_8 = l_Lean_Syntax_isOfKind(x_2, x_7); x_9 = lean_box(0); -x_10 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__6; +x_10 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__6; x_11 = lean_st_mk_ref(x_10, x_6); if (x_8 == 0) { @@ -15269,8 +15418,8 @@ if (x_12 == 0) lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_dec(x_2); lean_dec(x_1); -x_15 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__2; -x_16 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__3; +x_15 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__2; +x_16 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__3; x_17 = l_Lean_throwError___at_Lean_Meta_setInlineAttribute___spec__1(x_15, x_16, x_13, x_4, x_5, x_14); lean_dec(x_5); lean_dec(x_4); @@ -15311,8 +15460,8 @@ lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; lean_dec(x_23); lean_dec(x_2); lean_dec(x_1); -x_26 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__2; -x_27 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__3; +x_26 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__2; +x_27 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__3; x_28 = l_Lean_throwError___at_Lean_Meta_setInlineAttribute___spec__1(x_26, x_27, x_13, x_4, x_5, x_14); lean_dec(x_5); lean_dec(x_4); @@ -15342,7 +15491,7 @@ lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; x_33 = lean_unsigned_to_nat(0u); x_34 = l_Lean_Syntax_getArg(x_23, x_33); lean_dec(x_23); -x_35 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__8; +x_35 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__8; lean_inc(x_34); x_36 = l_Lean_Syntax_isOfKind(x_34, x_35); if (x_36 == 0) @@ -15351,8 +15500,8 @@ lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; lean_dec(x_34); lean_dec(x_2); lean_dec(x_1); -x_37 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__2; -x_38 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__3; +x_37 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__2; +x_38 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__3; x_39 = l_Lean_throwError___at_Lean_Meta_setInlineAttribute___spec__1(x_37, x_38, x_13, x_4, x_5, x_14); lean_dec(x_5); lean_dec(x_4); @@ -15385,9 +15534,9 @@ lean_dec(x_34); x_46 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_46, 0, x_45); x_47 = lean_box(0); -x_48 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__3; +x_48 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__3; lean_inc(x_13); -x_49 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10(x_2, x_9, x_3, x_1, x_47, x_46, x_48, x_13, x_4, x_5, x_14); +x_49 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10(x_2, x_9, x_3, x_1, x_47, x_46, x_48, x_13, x_4, x_5, x_14); lean_dec(x_46); if (lean_obj_tag(x_49) == 0) { @@ -15451,9 +15600,9 @@ else lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_dec(x_23); x_61 = lean_box(0); -x_62 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__3; +x_62 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__3; lean_inc(x_13); -x_63 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10(x_2, x_9, x_3, x_1, x_61, x_9, x_62, x_13, x_4, x_5, x_14); +x_63 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10(x_2, x_9, x_3, x_1, x_61, x_9, x_62, x_13, x_4, x_5, x_14); if (lean_obj_tag(x_63) == 0) { lean_object* x_64; lean_object* x_65; lean_object* x_66; uint8_t x_67; @@ -15513,14 +15662,14 @@ return x_74; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__12(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__12(lean_object* x_1, lean_object* x_2) { _start: { lean_inc(x_1); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__13(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__13(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; @@ -15537,7 +15686,7 @@ x_9 = l_Lean_Elab_Tactic_Ext_instInhabitedExtTheorems; x_10 = l_Lean_Elab_Tactic_Ext_getExtTheorems___closed__1; x_11 = l_Lean_ScopedEnvExtension_getState___rarg(x_9, x_10, x_8); lean_dec(x_8); -x_12 = l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__8(x_11, x_1, x_2, x_3, x_7); +x_12 = l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__8(x_11, x_1, x_2, x_3, x_7); if (lean_obj_tag(x_12) == 0) { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; @@ -15559,10 +15708,10 @@ lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean x_19 = lean_ctor_get(x_16, 0); x_20 = lean_ctor_get(x_16, 4); lean_dec(x_20); -x_21 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__12___boxed), 2, 1); +x_21 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__12___boxed), 2, 1); lean_closure_set(x_21, 0, x_13); x_22 = l_Lean_ScopedEnvExtension_modifyState___rarg(x_10, x_19, x_21); -x_23 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__2; +x_23 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__2; lean_ctor_set(x_16, 4, x_23); lean_ctor_set(x_16, 0, x_22); x_24 = lean_st_ref_set(x_3, x_16, x_17); @@ -15605,10 +15754,10 @@ lean_inc(x_33); lean_inc(x_32); lean_inc(x_31); lean_dec(x_16); -x_37 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__12___boxed), 2, 1); +x_37 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__12___boxed), 2, 1); lean_closure_set(x_37, 0, x_13); x_38 = l_Lean_ScopedEnvExtension_modifyState___rarg(x_10, x_31, x_37); -x_39 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__2; +x_39 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__2; x_40 = lean_alloc_ctor(0, 7, 0); lean_ctor_set(x_40, 0, x_38); lean_ctor_set(x_40, 1, x_32); @@ -15663,7 +15812,7 @@ return x_49; } } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -15673,37 +15822,37 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__1; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__1; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__1; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__2; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__2; x_2 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__10; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__3; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__2; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__3; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__5() { _start: { lean_object* x_1; @@ -15711,17 +15860,17 @@ x_1 = lean_mk_string_unchecked("initFn", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__6() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__4; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__5; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__4; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__5; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__7() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__7() { _start: { lean_object* x_1; @@ -15729,57 +15878,57 @@ x_1 = lean_mk_string_unchecked("_@", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__8() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__6; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__7; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__6; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__7; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__9() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__8; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__8; x_2 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__10() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__9; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__1; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__9; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__11() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__10; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__10; x_2 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__10; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__12() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__11; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__2; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__11; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__13() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__13() { _start: { lean_object* x_1; @@ -15787,27 +15936,27 @@ x_1 = lean_mk_string_unchecked("_hyg", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__14() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__12; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__13; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__12; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__13; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__15() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__14; -x_2 = lean_unsigned_to_nat(3766u); +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__14; +x_2 = lean_unsigned_to_nat(3660u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__16() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__16() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -15817,7 +15966,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__17() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__17() { _start: { lean_object* x_1; @@ -15825,13 +15974,13 @@ x_1 = lean_mk_string_unchecked("Marks a theorem as an extensionality theorem", 4 return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__18() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__18() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__15; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__16; -x_3 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__17; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__15; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__16; +x_3 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__17; x_4 = 0; x_5 = lean_alloc_ctor(0, 3, 1); lean_ctor_set(x_5, 0, x_1); @@ -15841,29 +15990,29 @@ lean_ctor_set_uint8(x_5, sizeof(void*)*3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__19() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__19() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___boxed), 6, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___boxed), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__20() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__20() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__13___boxed), 4, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__13___boxed), 4, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__21() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__21() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__18; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__19; -x_3 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__20; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__18; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__19; +x_3 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__20; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -15871,120 +16020,120 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__21; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__21; x_3 = l_Lean_registerBuiltinAttribute(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_throwError___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__3(x_1, x_2, x_3, x_4); +x_5 = l_Lean_throwError___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__3(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; -x_6 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__2(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__2(x_1, x_2, x_3, x_4, x_5); lean_dec(x_4); lean_dec(x_1); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4(x_1, x_2, x_3, x_4); +x_5 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4(x_1, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_2); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__5___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5(x_1, x_2); +x_3 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__5(x_1, x_2); lean_dec(x_2); lean_dec(x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__1(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__1___lambda__1(x_1, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_1); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__1___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__2(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__1___lambda__2(x_1, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_2); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__1___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; -x_7 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__1___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_5); lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__1___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; -x_7 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__1___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_5); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__1(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_ScopedEnvExtension_add___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_ScopedEnvExtension_add___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { uint8_t x_9; lean_object* x_10; x_9 = lean_unbox(x_3); lean_dec(x_3); -x_10 = l_Lean_ScopedEnvExtension_add___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__6(x_1, x_2, x_9, x_4, x_5, x_6, x_7, x_8); +x_10 = l_Lean_ScopedEnvExtension_add___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__6(x_1, x_2, x_9, x_4, x_5, x_6, x_7, x_8); lean_dec(x_7); lean_dec(x_5); lean_dec(x_4); return x_10; } } -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; -x_8 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__7(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__7(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_6); lean_dec(x_4); lean_dec(x_3); @@ -15992,67 +16141,67 @@ lean_dec(x_1); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__8___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__8___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; -x_7 = l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__8___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__8___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; -x_6 = l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__8(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__8(x_1, x_2, x_3, x_4, x_5); lean_dec(x_4); lean_dec(x_3); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__1(x_1, x_2, x_3); +x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__1(x_1, x_2, x_3); lean_dec(x_2); lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__2(x_1, x_2, x_3); +x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__2(x_1, x_2, x_3); lean_dec(x_2); lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3(x_1, x_2, x_3); +x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__3(x_1, x_2, x_3); lean_dec(x_2); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; -x_6 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__5(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__5(x_1, x_2, x_3, x_4, x_5); lean_dec(x_4); lean_dec(x_1); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { uint8_t x_13; uint8_t x_14; lean_object* x_15; @@ -16060,12 +16209,12 @@ x_13 = lean_unbox(x_4); lean_dec(x_4); x_14 = lean_unbox(x_5); lean_dec(x_5); -x_15 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6(x_1, x_2, x_3, x_13, x_14, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_15 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6(x_1, x_2, x_3, x_13, x_14, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_7); return x_15; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { uint8_t x_13; uint8_t x_14; lean_object* x_15; @@ -16073,74 +16222,74 @@ x_13 = lean_unbox(x_3); lean_dec(x_3); x_14 = lean_unbox(x_4); lean_dec(x_4); -x_15 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_15 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__7(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_7); lean_dec(x_1); return x_15; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { uint8_t x_7; lean_object* x_8; x_7 = lean_unbox(x_3); lean_dec(x_3); -x_8 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__8(x_1, x_2, x_7, x_4, x_5, x_6); +x_8 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__8(x_1, x_2, x_7, x_4, x_5, x_6); lean_dec(x_5); lean_dec(x_1); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { uint8_t x_13; lean_object* x_14; x_13 = lean_unbox(x_3); lean_dec(x_3); -x_14 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9(x_1, x_2, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_14 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__9(x_1, x_2, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); return x_14; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { uint8_t x_12; lean_object* x_13; x_12 = lean_unbox(x_3); lean_dec(x_3); -x_13 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10(x_1, x_2, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_13 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10(x_1, x_2, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_6); lean_dec(x_5); return x_13; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { uint8_t x_7; lean_object* x_8; x_7 = lean_unbox(x_3); lean_dec(x_3); -x_8 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11(x_1, x_2, x_7, x_4, x_5, x_6); +x_8 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11(x_1, x_2, x_7, x_4, x_5, x_6); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__12___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__12___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__12(x_1, x_2); +x_3 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__12(x_1, x_2); lean_dec(x_2); lean_dec(x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__13(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__13(x_1, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_2); return x_5; @@ -17662,9 +17811,9 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheore { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__1; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__1; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__1; x_3 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__10; -x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__2; +x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__2; x_5 = l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheorem__1___closed__1; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -17683,9 +17832,9 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheore { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__1; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__1; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__1; x_3 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__10; -x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__2; +x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__2; x_5 = l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheorem__1___closed__3; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -20462,9 +20611,9 @@ static lean_object* _init_l_Lean_Elab_Tactic_Ext_evalExt___closed__1() { { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__1; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__1; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__1; x_3 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__10; -x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__2; +x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__2; x_5 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__5___closed__1; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -20635,9 +20784,9 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Ext_evalExt__1___close { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__1; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__1; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__1; x_3 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__10; -x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__2; +x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__2; x_5 = l___regBuiltin_Lean_Elab_Tactic_Ext_evalExt__1___closed__1; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -20886,16 +21035,16 @@ l_Lean_getConstInfoInduct___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__1_ lean_mark_persistent(l_Lean_getConstInfoInduct___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__1___closed__3); l_Lean_getConstInfoInduct___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__1___closed__4 = _init_l_Lean_getConstInfoInduct___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__1___closed__4(); lean_mark_persistent(l_Lean_getConstInfoInduct___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__1___closed__4); -l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__1 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__1(); -lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__1); -l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__2 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__2(); -lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__2); -l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__3 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__3(); -lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__3); -l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__4 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__4(); -lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__4); -l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5(); -lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5); +l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__1 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__1(); +lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__1); +l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__2 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__2(); +lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__2); +l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__3 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__3(); +lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__3); +l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__4 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__4(); +lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__4); +l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5(); +lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5); l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__1 = _init_l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__1(); lean_mark_persistent(l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__1); l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__2 = _init_l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__2(); @@ -20984,6 +21133,10 @@ l_Lean_Elab_Tactic_Ext_realizeExtTheorem___closed__1 = _init_l_Lean_Elab_Tactic_ lean_mark_persistent(l_Lean_Elab_Tactic_Ext_realizeExtTheorem___closed__1); l_Lean_Elab_Tactic_Ext_realizeExtTheorem___closed__2 = _init_l_Lean_Elab_Tactic_Ext_realizeExtTheorem___closed__2(); lean_mark_persistent(l_Lean_Elab_Tactic_Ext_realizeExtTheorem___closed__2); +l_Lean_getConstInfo___at_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___spec__1___closed__1 = _init_l_Lean_getConstInfo___at_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___spec__1___closed__1(); +lean_mark_persistent(l_Lean_getConstInfo___at_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___spec__1___closed__1); +l_Lean_getConstInfo___at_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___spec__1___closed__2 = _init_l_Lean_getConstInfo___at_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___spec__1___closed__2(); +lean_mark_persistent(l_Lean_getConstInfo___at_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___spec__1___closed__2); l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__1 = _init_l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__1(); lean_mark_persistent(l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__1); l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__2(); @@ -21130,66 +21283,66 @@ l_Lean_Elab_Tactic_Ext_instInhabitedExtTheorem___closed__1 = _init_l_Lean_Elab_T lean_mark_persistent(l_Lean_Elab_Tactic_Ext_instInhabitedExtTheorem___closed__1); l_Lean_Elab_Tactic_Ext_instInhabitedExtTheorem = _init_l_Lean_Elab_Tactic_Ext_instInhabitedExtTheorem(); lean_mark_persistent(l_Lean_Elab_Tactic_Ext_instInhabitedExtTheorem); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__1 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__1(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__1); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__2 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__2(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__2); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__3 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__3(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__3); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__4 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__4(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__4); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__5 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__5(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__5); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__6 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__6(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__6); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__7 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__7(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__7); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__8 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__8(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__8); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__9 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__9(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__9); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__10 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__10(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__10); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__11 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__11(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__11); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__12 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__12(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__12); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__13 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__13(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__13); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__14 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__14(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__14); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__15 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__15(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__15); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__16 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__16(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__16); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__17 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__17(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__17); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__18 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__18(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__18); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__19 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__19(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__19); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__20 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__20(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__20); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__21 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__21(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__21); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__22 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__22(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__22); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__23 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__23(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__23); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__24 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__24(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__24); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__25 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__25(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__25); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__26 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__26(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__26); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__27 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__27(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__27); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__28 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__28(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__28); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__29 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__29(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__29); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__30 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__30(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__30); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__1 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__1(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__1); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__2 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__2(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__2); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__3 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__3(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__3); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__4 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__4(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__4); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__5 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__5(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__5); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__6 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__6(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__6); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__7 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__7(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__7); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__8 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__8(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__8); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__9 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__9(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__9); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__10 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__10(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__10); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__11 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__11(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__11); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__12 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__12(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__12); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__13 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__13(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__13); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__14 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__14(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__14); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__15 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__15(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__15); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__16 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__16(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__16); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__17 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__17(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__17); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__18 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__18(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__18); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__19 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__19(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__19); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__20 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__20(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__20); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__21 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__21(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__21); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__22 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__22(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__22); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__23 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__23(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__23); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__24 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__24(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__24); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__25 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__25(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__25); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__26 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__26(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__26); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__27 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__27(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__27); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__28 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__28(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__28); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__29 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__29(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__29); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__30 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__30(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3085____closed__30); l_Lean_Elab_Tactic_Ext_instReprExtTheorem___closed__1 = _init_l_Lean_Elab_Tactic_Ext_instReprExtTheorem___closed__1(); lean_mark_persistent(l_Lean_Elab_Tactic_Ext_instReprExtTheorem___closed__1); l_Lean_Elab_Tactic_Ext_instReprExtTheorem = _init_l_Lean_Elab_Tactic_Ext_instReprExtTheorem(); @@ -21210,37 +21363,37 @@ l_Lean_Elab_Tactic_Ext_extExt_config___closed__1 = _init_l_Lean_Elab_Tactic_Ext_ lean_mark_persistent(l_Lean_Elab_Tactic_Ext_extExt_config___closed__1); l_Lean_Elab_Tactic_Ext_extExt_config = _init_l_Lean_Elab_Tactic_Ext_extExt_config(); lean_mark_persistent(l_Lean_Elab_Tactic_Ext_extExt_config); -l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3___closed__1 = _init_l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3___closed__1(); -l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3___closed__2 = _init_l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3___closed__2(); -l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__6___closed__1 = _init_l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__6___closed__1(); -lean_mark_persistent(l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__6___closed__1); -l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9___closed__1 = _init_l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9___closed__1(); -lean_mark_persistent(l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9___closed__1); -l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__13___closed__1 = _init_l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__13___closed__1(); -lean_mark_persistent(l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__13___closed__1); -l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__1 = _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__1(); -lean_mark_persistent(l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__1); -l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__2 = _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__2(); -lean_mark_persistent(l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__2); -l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__3 = _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__3(); -lean_mark_persistent(l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__3); -l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__4 = _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__4(); -lean_mark_persistent(l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__4); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__1 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__1); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__2 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__2); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__3 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__3); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__4 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__4); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__5 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__5); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__6 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__6); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__7 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__7); -if (builtin) {res = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471_(lean_io_mk_world()); +l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__3___closed__1 = _init_l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__3___closed__1(); +l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__3___closed__2 = _init_l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__3___closed__2(); +l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__6___closed__1 = _init_l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__6___closed__1(); +lean_mark_persistent(l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__6___closed__1); +l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__9___closed__1 = _init_l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__9___closed__1(); +lean_mark_persistent(l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__9___closed__1); +l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__13___closed__1 = _init_l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__13___closed__1(); +lean_mark_persistent(l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__13___closed__1); +l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__1___closed__1 = _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__1___closed__1(); +lean_mark_persistent(l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__1___closed__1); +l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__1___closed__2 = _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__1___closed__2(); +lean_mark_persistent(l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__1___closed__2); +l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__1___closed__3 = _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__1___closed__3(); +lean_mark_persistent(l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__1___closed__3); +l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__1___closed__4 = _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__1___closed__4(); +lean_mark_persistent(l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____spec__1___closed__4); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__1 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__1); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__2 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__2); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__3 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__3); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__4 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__4); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__5 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__5); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__6 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__6); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__7 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365____closed__7); +if (builtin) {res = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3365_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_Elab_Tactic_Ext_extExtension = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Elab_Tactic_Ext_extExtension); @@ -21253,119 +21406,119 @@ l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___rarg___closed__1 = _init_l_Lean_Elab_ lean_mark_persistent(l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___rarg___closed__1); l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___rarg___closed__2 = _init_l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___rarg___closed__2(); lean_mark_persistent(l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___rarg___closed__2); -l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__1 = _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__1(); -lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__1); -l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__2 = _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__2(); -lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__2); -l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__3 = _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__3(); -lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__3); -l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__4 = _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__4(); -lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__4); -l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__5 = _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__5(); -lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__5); -l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__6 = _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__6(); -lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__6); -l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___rarg___closed__1 = _init_l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___rarg___closed__1(); -lean_mark_persistent(l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___rarg___closed__1); -l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___rarg___closed__2 = _init_l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___rarg___closed__2(); -lean_mark_persistent(l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___rarg___closed__2); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__1 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__1); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__2 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__2); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__3 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__3); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__1 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__1); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__2 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__2); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__3 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__3); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__4 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__4); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__5 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__5); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__6 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__6); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__7 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__7); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7___closed__1 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7___closed__1); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7___closed__2 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7___closed__2); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9___closed__1 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9___closed__1); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9___closed__2 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9___closed__2); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__1 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__1); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__2 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__2); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__3 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__3); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__4 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__4); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__5 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__5); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__1 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__1); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__2 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__2); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__3 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__3); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__4 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__4); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__5 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__5); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__6 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__6); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__7 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__7); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__8 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__8(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__8); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__1 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__1); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__2 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__2); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__3 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__3); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__4 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__4); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__5 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__5); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__6 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__6); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__7 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__7); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__8 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__8(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__8); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__9 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__9(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__9); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__10 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__10(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__10); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__11 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__11(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__11); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__12 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__12(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__12); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__13 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__13(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__13); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__14 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__14(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__14); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__15 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__15(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__15); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__16 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__16(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__16); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__17 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__17(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__17); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__18 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__18(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__18); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__19 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__19(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__19); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__20 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__20(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__20); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__21 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__21(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__21); -if (builtin) {res = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766_(lean_io_mk_world()); +l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__1 = _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__1(); +lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__1); +l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__2 = _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__2(); +lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__2); +l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__3 = _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__3(); +lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__3); +l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__4 = _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__4(); +lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__4); +l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__5 = _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__5(); +lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__5); +l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__6 = _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__6(); +lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__4___closed__6); +l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__5___rarg___closed__1 = _init_l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__5___rarg___closed__1(); +lean_mark_persistent(l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__5___rarg___closed__1); +l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__5___rarg___closed__2 = _init_l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__5___rarg___closed__2(); +lean_mark_persistent(l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____spec__5___rarg___closed__2); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__3___closed__1 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__3___closed__1); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__3___closed__2 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__3___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__3___closed__2); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__3___closed__3 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__3___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__3___closed__3); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__1 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__1); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__2 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__2); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__3 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__3); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__4 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__4); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__5 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__5); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__6 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__6); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__7 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__6___closed__7); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__7___closed__1 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__7___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__7___closed__1); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__7___closed__2 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__7___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__7___closed__2); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__9___closed__1 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__9___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__9___closed__1); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__9___closed__2 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__9___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__9___closed__2); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__1 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__1); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__2 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__2); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__3 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__3); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__4 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__4); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__5 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__10___closed__5); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__1 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__1); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__2 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__2); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__3 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__3); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__4 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__4); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__5 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__5); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__6 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__6); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__7 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__7); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__8 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__8(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____lambda__11___closed__8); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__1 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__1); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__2 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__2); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__3 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__3); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__4 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__4); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__5 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__5); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__6 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__6); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__7 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__7); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__8 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__8(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__8); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__9 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__9(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__9); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__10 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__10(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__10); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__11 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__11(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__11); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__12 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__12(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__12); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__13 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__13(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__13); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__14 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__14(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__14); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__15 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__15(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__15); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__16 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__16(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__16); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__17 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__17(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__17); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__18 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__18(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__18); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__19 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__19(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__19); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__20 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__20(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__20); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__21 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__21(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660____closed__21); +if (builtin) {res = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3660_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_applyExtTheoremAt___spec__1___lambda__1___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_applyExtTheoremAt___spec__1___lambda__1___closed__1(); diff --git a/stage0/stdlib/Lean/Elab/Tactic/Generalize.c b/stage0/stdlib/Lean/Elab/Tactic/Generalize.c index 1863e35acadf..5fddcfbf9d16 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/Generalize.c +++ b/stage0/stdlib/Lean/Elab/Tactic/Generalize.c @@ -16,6 +16,9 @@ extern "C" { static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalGeneralize_declRange__1___closed__3; lean_object* l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalGeneralize__1(lean_object*); +static lean_object* l_Lean_getLocalHyps___at_Lean_Elab_Tactic_evalGeneralize___spec__3___closed__1; +LEAN_EXPORT lean_object* l_Lean_getLocalHyps___at_Lean_Elab_Tactic_evalGeneralize___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_forInUnsafe_loop___at_Lean_Elab_Tactic_evalGeneralize___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* l_Lean_Elab_Tactic_expandOptLocation(lean_object*); lean_object* l_Lean_Syntax_getId(lean_object*); extern lean_object* l_Lean_Elab_Tactic_tacticElabAttribute; @@ -23,28 +26,38 @@ lean_object* lean_array_push(lean_object*, lean_object*); lean_object* l_Array_toSubarray___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalGeneralize___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalGeneralize_declRange__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_PersistentArray_forInAux___at_Lean_Elab_Tactic_evalGeneralize___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*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalGeneralize__1___closed__3; lean_object* lean_array_fget(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_evalGeneralize___closed__3; 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_object* l_Lean_Expr_fvarId_x21(lean_object*); lean_object* l_Lean_addBuiltinDeclarationRanges(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalGeneralize___boxed__const__1; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalGeneralize___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_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalGeneralize___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalGeneralize___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_getFVarIds(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalGeneralize___spec__7(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_evalGeneralize___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalGeneralize__1___closed__6; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalGeneralize__1___closed__1; lean_object* l_Lean_Elab_Tactic_elabTerm(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalGeneralize_declRange__1___closed__2; +LEAN_EXPORT lean_object* l_Lean_PersistentArray_forIn___at_Lean_Elab_Tactic_evalGeneralize___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_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalGeneralize___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_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalGeneralize___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentArray_forIn___at_Lean_Elab_Tactic_evalGeneralize___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_EXPORT lean_object* l_Lean_PersistentArray_forIn___at_Lean_Elab_Tactic_evalGeneralize___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* 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_getLocalHyps___at_Lean_Elab_Tactic_evalGeneralize___spec__3(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_evalGeneralize_declRange__1___closed__5; +LEAN_EXPORT lean_object* l_Lean_PersistentArray_forIn___at_Lean_Elab_Tactic_evalGeneralize___spec__4___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MVarId_withContext___at_Lean_Elab_Tactic_withMainContext___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MVarId_generalizeHyp(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalGeneralize__1___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalGeneralize__1___closed__8; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalGeneralize(lean_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_evalGeneralize___spec__9___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getSepArgs(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalGeneralize___lambda__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_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalGeneralize__1___closed__4; @@ -52,12 +65,15 @@ lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalGeneralize_declRange__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalGeneralize___lambda__2___boxed(lean_object**); lean_object* l_Array_append___rarg(lean_object*, lean_object*); +uint8_t l_Lean_LocalDecl_isImplementationDetail(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalGeneralize___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalGeneralize__1___closed__10; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalGeneralize__1___closed__9; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalGeneralize__1___closed__7; lean_object* l_Lean_Elab_Term_addLocalVarInfo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalGeneralize___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_PersistentArray_forInAux___at_Lean_Elab_Tactic_evalGeneralize___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentArray_forInAux___at_Lean_Elab_Tactic_evalGeneralize___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_EXPORT lean_object* l_Lean_Elab_Tactic_evalGeneralize___lambda__2(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*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_evalGeneralize___closed__1; @@ -66,22 +82,27 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalGeneralize___lambda__3___boxed(l static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalGeneralize_declRange__1___closed__7; lean_object* lean_array_mk(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalGeneralize__1___closed__5; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalGeneralize___spec__8(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalGeneralize___lambda__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*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalGeneralize___spec__9(size_t, size_t, lean_object*); lean_object* lean_array_uget(lean_object*, size_t); lean_object* l_Lean_Expr_fvar___override(lean_object*); size_t lean_array_size(lean_object*); lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalGeneralize_declRange__1___closed__4; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalGeneralize___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_array_get_size(lean_object*); +lean_object* l_Lean_LocalDecl_toExpr(lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); -lean_object* l_Lean_LocalContext_getFVarIds(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalGeneralize___lambda__3(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_nat_add(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalGeneralize___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_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalGeneralize___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_array_uset(lean_object*, size_t, lean_object*); lean_object* l_Lean_Elab_Tactic_replaceMainGoal(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalGeneralize_declRange__1___closed__6; +LEAN_EXPORT lean_object* l_Lean_PersistentArray_forInAux___at_Lean_Elab_Tactic_evalGeneralize___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalGeneralize___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { @@ -630,6 +651,758 @@ return x_52; } } } +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalGeneralize___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, lean_object* x_14, lean_object* x_15) { +_start: +{ +uint8_t x_16; +x_16 = lean_usize_dec_lt(x_5, x_4); +if (x_16 == 0) +{ +lean_object* x_17; +lean_dec(x_2); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_6); +lean_ctor_set(x_17, 1, x_15); +return x_17; +} +else +{ +lean_object* x_18; uint8_t x_19; +x_18 = lean_array_uget(x_3, x_5); +x_19 = !lean_is_exclusive(x_6); +if (x_19 == 0) +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_20 = lean_ctor_get(x_6, 1); +x_21 = lean_ctor_get(x_6, 0); +lean_dec(x_21); +lean_inc(x_20); +x_22 = l_Lean_PersistentArray_forInAux___at_Lean_Elab_Tactic_evalGeneralize___spec__5(x_1, x_18, x_20, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +lean_dec(x_18); +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +if (lean_obj_tag(x_23) == 0) +{ +uint8_t x_24; +lean_dec(x_2); +x_24 = !lean_is_exclusive(x_22); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; +x_25 = lean_ctor_get(x_22, 0); +lean_dec(x_25); +x_26 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_26, 0, x_23); +lean_ctor_set(x_6, 0, x_26); +lean_ctor_set(x_22, 0, x_6); +return x_22; +} +else +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_22, 1); +lean_inc(x_27); +lean_dec(x_22); +x_28 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_28, 0, x_23); +lean_ctor_set(x_6, 0, x_28); +x_29 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_29, 0, x_6); +lean_ctor_set(x_29, 1, x_27); +return x_29; +} +} +else +{ +lean_object* x_30; lean_object* x_31; size_t x_32; size_t x_33; +lean_dec(x_20); +x_30 = lean_ctor_get(x_22, 1); +lean_inc(x_30); +lean_dec(x_22); +x_31 = lean_ctor_get(x_23, 0); +lean_inc(x_31); +lean_dec(x_23); +lean_inc(x_2); +lean_ctor_set(x_6, 1, x_31); +lean_ctor_set(x_6, 0, x_2); +x_32 = 1; +x_33 = lean_usize_add(x_5, x_32); +x_5 = x_33; +x_15 = x_30; +goto _start; +} +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_6, 1); +lean_inc(x_35); +lean_dec(x_6); +lean_inc(x_35); +x_36 = l_Lean_PersistentArray_forInAux___at_Lean_Elab_Tactic_evalGeneralize___spec__5(x_1, x_18, x_35, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +lean_dec(x_18); +x_37 = lean_ctor_get(x_36, 0); +lean_inc(x_37); +if (lean_obj_tag(x_37) == 0) +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; +lean_dec(x_2); +x_38 = lean_ctor_get(x_36, 1); +lean_inc(x_38); +if (lean_is_exclusive(x_36)) { + lean_ctor_release(x_36, 0); + lean_ctor_release(x_36, 1); + x_39 = x_36; +} else { + lean_dec_ref(x_36); + x_39 = lean_box(0); +} +x_40 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_40, 0, x_37); +x_41 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_41, 0, x_40); +lean_ctor_set(x_41, 1, x_35); +if (lean_is_scalar(x_39)) { + x_42 = lean_alloc_ctor(0, 2, 0); +} else { + x_42 = x_39; +} +lean_ctor_set(x_42, 0, x_41); +lean_ctor_set(x_42, 1, x_38); +return x_42; +} +else +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; size_t x_46; size_t x_47; +lean_dec(x_35); +x_43 = lean_ctor_get(x_36, 1); +lean_inc(x_43); +lean_dec(x_36); +x_44 = lean_ctor_get(x_37, 0); +lean_inc(x_44); +lean_dec(x_37); +lean_inc(x_2); +x_45 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_45, 0, x_2); +lean_ctor_set(x_45, 1, x_44); +x_46 = 1; +x_47 = lean_usize_add(x_5, x_46); +x_5 = x_47; +x_6 = x_45; +x_15 = x_43; +goto _start; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalGeneralize___spec__7(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_object* x_13, lean_object* x_14) { +_start: +{ +uint8_t x_15; +x_15 = lean_usize_dec_lt(x_4, x_3); +if (x_15 == 0) +{ +lean_object* x_16; +lean_dec(x_1); +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_5); +lean_ctor_set(x_16, 1, x_14); +return x_16; +} +else +{ +lean_object* x_17; +x_17 = lean_array_uget(x_2, x_4); +if (lean_obj_tag(x_17) == 0) +{ +uint8_t x_18; +x_18 = !lean_is_exclusive(x_5); +if (x_18 == 0) +{ +lean_object* x_19; size_t x_20; size_t x_21; +x_19 = lean_ctor_get(x_5, 0); +lean_dec(x_19); +lean_inc(x_1); +lean_ctor_set(x_5, 0, x_1); +x_20 = 1; +x_21 = lean_usize_add(x_4, x_20); +x_4 = x_21; +goto _start; +} +else +{ +lean_object* x_23; lean_object* x_24; size_t x_25; size_t x_26; +x_23 = lean_ctor_get(x_5, 1); +lean_inc(x_23); +lean_dec(x_5); +lean_inc(x_1); +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_1); +lean_ctor_set(x_24, 1, x_23); +x_25 = 1; +x_26 = lean_usize_add(x_4, x_25); +x_4 = x_26; +x_5 = x_24; +goto _start; +} +} +else +{ +uint8_t x_28; +x_28 = !lean_is_exclusive(x_5); +if (x_28 == 0) +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; +x_29 = lean_ctor_get(x_5, 1); +x_30 = lean_ctor_get(x_5, 0); +lean_dec(x_30); +x_31 = lean_ctor_get(x_17, 0); +lean_inc(x_31); +lean_dec(x_17); +x_32 = l_Lean_LocalDecl_isImplementationDetail(x_31); +if (x_32 == 0) +{ +lean_object* x_33; lean_object* x_34; size_t x_35; size_t x_36; +x_33 = l_Lean_LocalDecl_toExpr(x_31); +lean_dec(x_31); +x_34 = lean_array_push(x_29, x_33); +lean_inc(x_1); +lean_ctor_set(x_5, 1, x_34); +lean_ctor_set(x_5, 0, x_1); +x_35 = 1; +x_36 = lean_usize_add(x_4, x_35); +x_4 = x_36; +goto _start; +} +else +{ +size_t x_38; size_t x_39; +lean_dec(x_31); +lean_inc(x_1); +lean_ctor_set(x_5, 0, x_1); +x_38 = 1; +x_39 = lean_usize_add(x_4, x_38); +x_4 = x_39; +goto _start; +} +} +else +{ +lean_object* x_41; lean_object* x_42; uint8_t x_43; +x_41 = lean_ctor_get(x_5, 1); +lean_inc(x_41); +lean_dec(x_5); +x_42 = lean_ctor_get(x_17, 0); +lean_inc(x_42); +lean_dec(x_17); +x_43 = l_Lean_LocalDecl_isImplementationDetail(x_42); +if (x_43 == 0) +{ +lean_object* x_44; lean_object* x_45; lean_object* x_46; size_t x_47; size_t x_48; +x_44 = l_Lean_LocalDecl_toExpr(x_42); +lean_dec(x_42); +x_45 = lean_array_push(x_41, x_44); +lean_inc(x_1); +x_46 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_46, 0, x_1); +lean_ctor_set(x_46, 1, x_45); +x_47 = 1; +x_48 = lean_usize_add(x_4, x_47); +x_4 = x_48; +x_5 = x_46; +goto _start; +} +else +{ +lean_object* x_50; size_t x_51; size_t x_52; +lean_dec(x_42); +lean_inc(x_1); +x_50 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_50, 0, x_1); +lean_ctor_set(x_50, 1, x_41); +x_51 = 1; +x_52 = lean_usize_add(x_4, x_51); +x_4 = x_52; +x_5 = x_50; +goto _start; +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentArray_forInAux___at_Lean_Elab_Tactic_evalGeneralize___spec__5___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; lean_object* x_13; +x_12 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_12, 0, x_1); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_11); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentArray_forInAux___at_Lean_Elab_Tactic_evalGeneralize___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +if (lean_obj_tag(x_2) == 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; lean_object* x_20; +x_13 = lean_ctor_get(x_2, 0); +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_3); +x_16 = lean_array_size(x_13); +x_17 = 0; +x_18 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalGeneralize___spec__6(x_1, x_14, x_13, x_16, x_17, 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_19, 0); +lean_inc(x_20); +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_18, 1); +lean_inc(x_21); +lean_dec(x_18); +x_22 = lean_ctor_get(x_19, 1); +lean_inc(x_22); +lean_dec(x_19); +x_23 = lean_box(0); +x_24 = l_Lean_PersistentArray_forInAux___at_Lean_Elab_Tactic_evalGeneralize___spec__5___lambda__1(x_22, x_23, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_21); +return x_24; +} +else +{ +uint8_t x_25; +lean_dec(x_19); +x_25 = !lean_is_exclusive(x_18); +if (x_25 == 0) +{ +lean_object* x_26; lean_object* x_27; +x_26 = lean_ctor_get(x_18, 0); +lean_dec(x_26); +x_27 = lean_ctor_get(x_20, 0); +lean_inc(x_27); +lean_dec(x_20); +lean_ctor_set(x_18, 0, x_27); +return x_18; +} +else +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_18, 1); +lean_inc(x_28); +lean_dec(x_18); +x_29 = lean_ctor_get(x_20, 0); +lean_inc(x_29); +lean_dec(x_20); +x_30 = lean_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 +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; size_t x_34; size_t x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_31 = lean_ctor_get(x_2, 0); +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_3); +x_34 = lean_array_size(x_31); +x_35 = 0; +x_36 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalGeneralize___spec__7(x_32, x_31, x_34, x_35, x_33, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_37 = lean_ctor_get(x_36, 0); +lean_inc(x_37); +x_38 = lean_ctor_get(x_37, 0); +lean_inc(x_38); +if (lean_obj_tag(x_38) == 0) +{ +lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_39 = lean_ctor_get(x_36, 1); +lean_inc(x_39); +lean_dec(x_36); +x_40 = lean_ctor_get(x_37, 1); +lean_inc(x_40); +lean_dec(x_37); +x_41 = lean_box(0); +x_42 = l_Lean_PersistentArray_forInAux___at_Lean_Elab_Tactic_evalGeneralize___spec__5___lambda__1(x_40, x_41, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_39); +return x_42; +} +else +{ +uint8_t x_43; +lean_dec(x_37); +x_43 = !lean_is_exclusive(x_36); +if (x_43 == 0) +{ +lean_object* x_44; lean_object* x_45; +x_44 = lean_ctor_get(x_36, 0); +lean_dec(x_44); +x_45 = lean_ctor_get(x_38, 0); +lean_inc(x_45); +lean_dec(x_38); +lean_ctor_set(x_36, 0, x_45); +return x_36; +} +else +{ +lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_46 = lean_ctor_get(x_36, 1); +lean_inc(x_46); +lean_dec(x_36); +x_47 = lean_ctor_get(x_38, 0); +lean_inc(x_47); +lean_dec(x_38); +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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalGeneralize___spec__8(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_object* x_13, lean_object* x_14) { +_start: +{ +uint8_t x_15; +x_15 = lean_usize_dec_lt(x_4, x_3); +if (x_15 == 0) +{ +lean_object* x_16; +lean_dec(x_1); +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_5); +lean_ctor_set(x_16, 1, x_14); +return x_16; +} +else +{ +lean_object* x_17; +x_17 = lean_array_uget(x_2, x_4); +if (lean_obj_tag(x_17) == 0) +{ +uint8_t x_18; +x_18 = !lean_is_exclusive(x_5); +if (x_18 == 0) +{ +lean_object* x_19; size_t x_20; size_t x_21; +x_19 = lean_ctor_get(x_5, 0); +lean_dec(x_19); +lean_inc(x_1); +lean_ctor_set(x_5, 0, x_1); +x_20 = 1; +x_21 = lean_usize_add(x_4, x_20); +x_4 = x_21; +goto _start; +} +else +{ +lean_object* x_23; lean_object* x_24; size_t x_25; size_t x_26; +x_23 = lean_ctor_get(x_5, 1); +lean_inc(x_23); +lean_dec(x_5); +lean_inc(x_1); +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_1); +lean_ctor_set(x_24, 1, x_23); +x_25 = 1; +x_26 = lean_usize_add(x_4, x_25); +x_4 = x_26; +x_5 = x_24; +goto _start; +} +} +else +{ +uint8_t x_28; +x_28 = !lean_is_exclusive(x_5); +if (x_28 == 0) +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; +x_29 = lean_ctor_get(x_5, 1); +x_30 = lean_ctor_get(x_5, 0); +lean_dec(x_30); +x_31 = lean_ctor_get(x_17, 0); +lean_inc(x_31); +lean_dec(x_17); +x_32 = l_Lean_LocalDecl_isImplementationDetail(x_31); +if (x_32 == 0) +{ +lean_object* x_33; lean_object* x_34; size_t x_35; size_t x_36; +x_33 = l_Lean_LocalDecl_toExpr(x_31); +lean_dec(x_31); +x_34 = lean_array_push(x_29, x_33); +lean_inc(x_1); +lean_ctor_set(x_5, 1, x_34); +lean_ctor_set(x_5, 0, x_1); +x_35 = 1; +x_36 = lean_usize_add(x_4, x_35); +x_4 = x_36; +goto _start; +} +else +{ +size_t x_38; size_t x_39; +lean_dec(x_31); +lean_inc(x_1); +lean_ctor_set(x_5, 0, x_1); +x_38 = 1; +x_39 = lean_usize_add(x_4, x_38); +x_4 = x_39; +goto _start; +} +} +else +{ +lean_object* x_41; lean_object* x_42; uint8_t x_43; +x_41 = lean_ctor_get(x_5, 1); +lean_inc(x_41); +lean_dec(x_5); +x_42 = lean_ctor_get(x_17, 0); +lean_inc(x_42); +lean_dec(x_17); +x_43 = l_Lean_LocalDecl_isImplementationDetail(x_42); +if (x_43 == 0) +{ +lean_object* x_44; lean_object* x_45; lean_object* x_46; size_t x_47; size_t x_48; +x_44 = l_Lean_LocalDecl_toExpr(x_42); +lean_dec(x_42); +x_45 = lean_array_push(x_41, x_44); +lean_inc(x_1); +x_46 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_46, 0, x_1); +lean_ctor_set(x_46, 1, x_45); +x_47 = 1; +x_48 = lean_usize_add(x_4, x_47); +x_4 = x_48; +x_5 = x_46; +goto _start; +} +else +{ +lean_object* x_50; size_t x_51; size_t x_52; +lean_dec(x_42); +lean_inc(x_1); +x_50 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_50, 0, x_1); +lean_ctor_set(x_50, 1, x_41); +x_51 = 1; +x_52 = lean_usize_add(x_4, x_51); +x_4 = x_52; +x_5 = x_50; +goto _start; +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentArray_forIn___at_Lean_Elab_Tactic_evalGeneralize___spec__4___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +x_12 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_1); +lean_ctor_set(x_12, 1, x_11); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentArray_forIn___at_Lean_Elab_Tactic_evalGeneralize___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) { +_start: +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_1, 0); +lean_inc(x_2); +x_13 = l_Lean_PersistentArray_forInAux___at_Lean_Elab_Tactic_evalGeneralize___spec__5(x_2, x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_2); +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +if (lean_obj_tag(x_14) == 0) +{ +uint8_t x_15; +x_15 = !lean_is_exclusive(x_13); +if (x_15 == 0) +{ +lean_object* x_16; lean_object* x_17; +x_16 = lean_ctor_get(x_13, 0); +lean_dec(x_16); +x_17 = lean_ctor_get(x_14, 0); +lean_inc(x_17); +lean_dec(x_14); +lean_ctor_set(x_13, 0, x_17); +return x_13; +} +else +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_13, 1); +lean_inc(x_18); +lean_dec(x_13); +x_19 = lean_ctor_get(x_14, 0); +lean_inc(x_19); +lean_dec(x_14); +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_19); +lean_ctor_set(x_20, 1, x_18); +return x_20; +} +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; size_t x_26; size_t x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_21 = lean_ctor_get(x_13, 1); +lean_inc(x_21); +lean_dec(x_13); +x_22 = lean_ctor_get(x_14, 0); +lean_inc(x_22); +lean_dec(x_14); +x_23 = lean_ctor_get(x_1, 1); +x_24 = lean_box(0); +x_25 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_25, 0, x_24); +lean_ctor_set(x_25, 1, x_22); +x_26 = lean_array_size(x_23); +x_27 = 0; +x_28 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalGeneralize___spec__8(x_24, x_23, x_26, x_27, x_25, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_21); +x_29 = lean_ctor_get(x_28, 0); +lean_inc(x_29); +x_30 = lean_ctor_get(x_29, 0); +lean_inc(x_30); +if (lean_obj_tag(x_30) == 0) +{ +uint8_t x_31; +x_31 = !lean_is_exclusive(x_28); +if (x_31 == 0) +{ +lean_object* x_32; lean_object* x_33; +x_32 = lean_ctor_get(x_28, 0); +lean_dec(x_32); +x_33 = lean_ctor_get(x_29, 1); +lean_inc(x_33); +lean_dec(x_29); +lean_ctor_set(x_28, 0, x_33); +return x_28; +} +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_28, 1); +lean_inc(x_34); +lean_dec(x_28); +x_35 = lean_ctor_get(x_29, 1); +lean_inc(x_35); +lean_dec(x_29); +x_36 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_36, 0, x_35); +lean_ctor_set(x_36, 1, x_34); +return x_36; +} +} +else +{ +uint8_t x_37; +lean_dec(x_29); +x_37 = !lean_is_exclusive(x_28); +if (x_37 == 0) +{ +lean_object* x_38; lean_object* x_39; +x_38 = lean_ctor_get(x_28, 0); +lean_dec(x_38); +x_39 = lean_ctor_get(x_30, 0); +lean_inc(x_39); +lean_dec(x_30); +lean_ctor_set(x_28, 0, x_39); +return x_28; +} +else +{ +lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_40 = lean_ctor_get(x_28, 1); +lean_inc(x_40); +lean_dec(x_28); +x_41 = lean_ctor_get(x_30, 0); +lean_inc(x_41); +lean_dec(x_30); +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; +} +} +} +} +} +static lean_object* _init_l_Lean_getLocalHyps___at_Lean_Elab_Tactic_evalGeneralize___spec__3___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_array_mk(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_getLocalHyps___at_Lean_Elab_Tactic_evalGeneralize___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_10 = lean_ctor_get(x_5, 1); +x_11 = lean_ctor_get(x_10, 1); +x_12 = l_Lean_getLocalHyps___at_Lean_Elab_Tactic_evalGeneralize___spec__3___closed__1; +x_13 = l_Lean_PersistentArray_forIn___at_Lean_Elab_Tactic_evalGeneralize___spec__4(x_11, x_12, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_14 = !lean_is_exclusive(x_13); +if (x_14 == 0) +{ +return x_13; +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_15 = lean_ctor_get(x_13, 0); +x_16 = lean_ctor_get(x_13, 1); +lean_inc(x_16); +lean_inc(x_15); +lean_dec(x_13); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_15); +lean_ctor_set(x_17, 1, x_16); +return x_17; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalGeneralize___spec__9(size_t x_1, size_t x_2, lean_object* x_3) { +_start: +{ +uint8_t x_4; +x_4 = lean_usize_dec_lt(x_2, x_1); +if (x_4 == 0) +{ +return x_3; +} +else +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; 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_Lean_Expr_fvarId_x21(x_5); +lean_dec(x_5); +x_9 = 1; +x_10 = lean_usize_add(x_2, x_9); +x_11 = lean_array_uset(x_7, x_2, x_8); +x_2 = x_10; +x_3 = x_11; +goto _start; +} +} +} LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalGeneralize___lambda__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_object* x_14, lean_object* x_15) { _start: { @@ -871,19 +1644,23 @@ x_25 = l_Lean_Elab_Tactic_expandOptLocation(x_24); lean_dec(x_24); if (lean_obj_tag(x_25) == 0) { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_11, 1); -lean_inc(x_26); -x_27 = l_Lean_LocalContext_getFVarIds(x_26); +lean_object* x_26; lean_object* x_27; lean_object* x_28; size_t x_29; lean_object* x_30; lean_object* x_31; +x_26 = l_Lean_getLocalHyps___at_Lean_Elab_Tactic_evalGeneralize___spec__3(x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_19); +x_27 = lean_ctor_get(x_26, 0); +lean_inc(x_27); +x_28 = lean_ctor_get(x_26, 1); +lean_inc(x_28); lean_dec(x_26); -x_28 = l_Lean_Elab_Tactic_evalGeneralize___lambda__3(x_20, x_22, x_21, x_3, x_5, x_27, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_19); -return x_28; +x_29 = lean_array_size(x_27); +x_30 = l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalGeneralize___spec__9(x_29, x_3, x_27); +x_31 = l_Lean_Elab_Tactic_evalGeneralize___lambda__3(x_20, x_22, x_21, x_3, x_5, x_30, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_28); +return x_31; } else { -lean_object* x_29; lean_object* x_30; -x_29 = lean_ctor_get(x_25, 0); -lean_inc(x_29); +lean_object* x_32; lean_object* x_33; +x_32 = lean_ctor_get(x_25, 0); +lean_inc(x_32); lean_dec(x_25); lean_inc(x_14); lean_inc(x_13); @@ -893,21 +1670,21 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -x_30 = l_Lean_Elab_Tactic_getFVarIds(x_29, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_19); -if (lean_obj_tag(x_30) == 0) +x_33 = l_Lean_Elab_Tactic_getFVarIds(x_32, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_19); +if (lean_obj_tag(x_33) == 0) { -lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_31 = lean_ctor_get(x_30, 0); -lean_inc(x_31); -x_32 = lean_ctor_get(x_30, 1); -lean_inc(x_32); -lean_dec(x_30); -x_33 = l_Lean_Elab_Tactic_evalGeneralize___lambda__3(x_20, x_22, x_21, x_3, x_5, x_31, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_32); -return x_33; +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 = l_Lean_Elab_Tactic_evalGeneralize___lambda__3(x_20, x_22, x_21, x_3, x_5, x_34, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_35); +return x_36; } else { -uint8_t x_34; +uint8_t x_37; lean_dec(x_22); lean_dec(x_21); lean_dec(x_20); @@ -920,30 +1697,30 @@ lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_5); -x_34 = !lean_is_exclusive(x_30); -if (x_34 == 0) +x_37 = !lean_is_exclusive(x_33); +if (x_37 == 0) { -return x_30; +return x_33; } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_35 = lean_ctor_get(x_30, 0); -x_36 = lean_ctor_get(x_30, 1); -lean_inc(x_36); -lean_inc(x_35); -lean_dec(x_30); -x_37 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -return x_37; +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_33, 0); +x_39 = lean_ctor_get(x_33, 1); +lean_inc(x_39); +lean_inc(x_38); +lean_dec(x_33); +x_40 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +return x_40; } } } } else { -uint8_t x_38; +uint8_t x_41; lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); @@ -953,23 +1730,23 @@ lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_5); -x_38 = !lean_is_exclusive(x_16); -if (x_38 == 0) +x_41 = !lean_is_exclusive(x_16); +if (x_41 == 0) { return x_16; } else { -lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_39 = lean_ctor_get(x_16, 0); -x_40 = lean_ctor_get(x_16, 1); -lean_inc(x_40); -lean_inc(x_39); +lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_42 = lean_ctor_get(x_16, 0); +x_43 = lean_ctor_get(x_16, 1); +lean_inc(x_43); +lean_inc(x_42); lean_dec(x_16); -x_41 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_41, 0, x_39); -lean_ctor_set(x_41, 1, x_40); -return x_41; +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; } } } @@ -978,28 +1755,19 @@ static lean_object* _init_l_Lean_Elab_Tactic_evalGeneralize___closed__1() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = lean_box(0); -x_2 = lean_array_mk(x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_evalGeneralize___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Tactic_evalGeneralize___closed__1; +x_1 = l_Lean_getLocalHyps___at_Lean_Elab_Tactic_evalGeneralize___spec__3___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_Elab_Tactic_evalGeneralize___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_evalGeneralize___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_evalGeneralize___closed__1; -x_2 = l_Lean_Elab_Tactic_evalGeneralize___closed__2; +x_1 = l_Lean_getLocalHyps___at_Lean_Elab_Tactic_evalGeneralize___spec__3___closed__1; +x_2 = l_Lean_Elab_Tactic_evalGeneralize___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); @@ -1025,7 +1793,7 @@ x_13 = l_Lean_Syntax_getArg(x_1, x_12); x_14 = l_Lean_Syntax_getSepArgs(x_13); lean_dec(x_13); x_15 = lean_array_size(x_14); -x_16 = l_Lean_Elab_Tactic_evalGeneralize___closed__3; +x_16 = l_Lean_Elab_Tactic_evalGeneralize___closed__2; x_17 = lean_box_usize(x_15); x_18 = l_Lean_Elab_Tactic_evalGeneralize___boxed__const__1; x_19 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalGeneralize___lambda__4___boxed), 15, 6); @@ -1076,6 +1844,167 @@ lean_dec(x_1); return x_16; } } +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalGeneralize___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +_start: +{ +size_t x_16; size_t x_17; lean_object* x_18; +x_16 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_17 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_18 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalGeneralize___spec__6(x_1, x_2, x_3, x_16, x_17, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_1); +return x_18; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalGeneralize___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +size_t x_15; size_t x_16; lean_object* x_17; +x_15 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_16 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_17 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalGeneralize___spec__7(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_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_2); +return x_17; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentArray_forInAux___at_Lean_Elab_Tactic_evalGeneralize___spec__5___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_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_PersistentArray_forInAux___at_Lean_Elab_Tactic_evalGeneralize___spec__5___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentArray_forInAux___at_Lean_Elab_Tactic_evalGeneralize___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: +{ +lean_object* x_13; +x_13 = l_Lean_PersistentArray_forInAux___at_Lean_Elab_Tactic_evalGeneralize___spec__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalGeneralize___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) { +_start: +{ +size_t x_15; size_t x_16; lean_object* x_17; +x_15 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_16 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_17 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalGeneralize___spec__8(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_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_2); +return x_17; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentArray_forIn___at_Lean_Elab_Tactic_evalGeneralize___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) { +_start: +{ +lean_object* x_12; +x_12 = l_Lean_PersistentArray_forIn___at_Lean_Elab_Tactic_evalGeneralize___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); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentArray_forIn___at_Lean_Elab_Tactic_evalGeneralize___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) { +_start: +{ +lean_object* x_12; +x_12 = l_Lean_PersistentArray_forIn___at_Lean_Elab_Tactic_evalGeneralize___spec__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +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_getLocalHyps___at_Lean_Elab_Tactic_evalGeneralize___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l_Lean_getLocalHyps___at_Lean_Elab_Tactic_evalGeneralize___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalGeneralize___spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; size_t x_5; lean_object* x_6; +x_4 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalGeneralize___spec__9(x_4, x_5, x_3); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalGeneralize___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, 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: { @@ -1375,12 +2304,12 @@ lean_dec_ref(res); res = initialize_Lean_Elab_Tactic_Location(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +l_Lean_getLocalHyps___at_Lean_Elab_Tactic_evalGeneralize___spec__3___closed__1 = _init_l_Lean_getLocalHyps___at_Lean_Elab_Tactic_evalGeneralize___spec__3___closed__1(); +lean_mark_persistent(l_Lean_getLocalHyps___at_Lean_Elab_Tactic_evalGeneralize___spec__3___closed__1); l_Lean_Elab_Tactic_evalGeneralize___closed__1 = _init_l_Lean_Elab_Tactic_evalGeneralize___closed__1(); lean_mark_persistent(l_Lean_Elab_Tactic_evalGeneralize___closed__1); l_Lean_Elab_Tactic_evalGeneralize___closed__2 = _init_l_Lean_Elab_Tactic_evalGeneralize___closed__2(); lean_mark_persistent(l_Lean_Elab_Tactic_evalGeneralize___closed__2); -l_Lean_Elab_Tactic_evalGeneralize___closed__3 = _init_l_Lean_Elab_Tactic_evalGeneralize___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_evalGeneralize___closed__3); l_Lean_Elab_Tactic_evalGeneralize___boxed__const__1 = _init_l_Lean_Elab_Tactic_evalGeneralize___boxed__const__1(); lean_mark_persistent(l_Lean_Elab_Tactic_evalGeneralize___boxed__const__1); l___regBuiltin_Lean_Elab_Tactic_evalGeneralize__1___closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_evalGeneralize__1___closed__1(); diff --git a/stage0/stdlib/Lean/Elab/Tactic/Induction.c b/stage0/stdlib/Lean/Elab/Tactic/Induction.c index 3ae273f9dec0..42a6d9278b7b 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/Induction.c +++ b/stage0/stdlib/Lean/Elab/Tactic/Induction.c @@ -19,7 +19,6 @@ lean_object* l_Lean_Elab_Tactic_tagUntaggedGoals(lean_object*, lean_object*, lea lean_object* l_Lean_Meta_getElimInfo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MVarId_isAssigned___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___lambda__3___closed__6; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137_(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_withAltsOfOptInductionAlts___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getAltNumFields___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapMAux___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -31,23 +30,23 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tac LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_expandCases_x3f(lean_object*); lean_object* l_Lean_Meta_getElimExprInfo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_format_pretty(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__12; +LEAN_EXPORT lean_object* l_Lean_Elab_Term_withNarrowedTacticReuse___at_Lean_Elab_Tactic_evalInduction___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getAltName(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_mkElimApp_loop___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutTacticIncrementality___at_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_ElimApp_setMotiveArg___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalInduction___lambda__1___boxed(lean_object**); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalAlt___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalInduction___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_mapMUnsafe_map___at_Lean_LocalContext_getFVars___spec__1(size_t, size_t, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalInduction_checkTargets___spec__1___closed__1; -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__1; static lean_object* l_Lean_Elab_Tactic_evalCases___lambda__4___closed__1; lean_object* l_Lean_Elab_Term_resolveId_x3f(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalCases_declRange__1___closed__1; lean_object* l_Lean_Meta_throwTacticEx___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079_(lean_object*); +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__6; lean_object* l_Lean_Elab_CommandContextInfo_save___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___spec__3___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getArgExpectedType(lean_object*); @@ -56,6 +55,7 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabCase LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_isMultiAlt___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_getInductiveValFromMajor___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*); +LEAN_EXPORT lean_object* l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalInduction___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalCases__1___closed__5; static lean_object* l_Lean_Elab_Tactic_elabCasesTargets___lambda__1___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalInduction__1___closed__2; @@ -79,7 +79,6 @@ static lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_g LEAN_EXPORT uint8_t l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_isMultiAlt(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_mkElimApp_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___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_generalizeVars(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalInduction___spec__3___lambda__1(lean_object*, lean_object*); lean_object* lean_io_promise_new(lean_object*); uint8_t l_Lean_Exception_isInterrupt(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*); @@ -94,7 +93,6 @@ static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalInduction_declRange__1__ lean_object* l_Lean_Elab_Tactic_evalTacticAt(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_withoutTacticIncrementality___at_Lean_Elab_Tactic_ElimApp_evalAlts_applyPreTac___spec__1___closed__1; static lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___closed__1; -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__10; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabCasesTargets___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_withAlwaysResolvedPromises___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalCases___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -108,6 +106,7 @@ lean_object* l_Lean_Syntax_getId(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_generalizeVars___spec__1___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_generalizeVars___spec__2(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Elab_Tactic_tacticElabAttribute; lean_object* l_Array_findIdx_x3f_loop___rarg(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__3; lean_object* l_Lean_Expr_sort___override(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutErrToSorry___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_elabTermForElim___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); @@ -127,9 +126,9 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tac lean_object* l_Lean_Meta_generalizeTargetsEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getAltNumFields___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_mkTacticInfo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__16; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getArgs(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_generalizeVars___spec__1___lambda__2___closed__3; lean_object* l___private_Lean_Meta_Tactic_Generalize_0__Lean_Meta_generalizeCore(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getFirstAltLhs(lean_object*); @@ -137,20 +136,20 @@ lean_object* l_Lean_Elab_Tactic_appendGoals(lean_object*, lean_object*, lean_obj LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___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* l_Lean_replaceRef(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___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*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___spec__5___at_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___spec__6___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_MVarId_assign___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*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_checkAltsOfOptInductionAlts(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__6; lean_object* lean_array_fget(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_casesOnSuffix; static lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___lambda__3___closed__4; static lean_object* l_Lean_Elab_Tactic_elabCasesTargets___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___spec__1(lean_object*, uint8_t, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_checkAltsOfOptInductionAlts___spec__1___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___spec__6(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__14; lean_object* l_Lean_Elab_Tactic_getMainGoal(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_elabTermForElim___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_FVarSubst_get(lean_object*, lean_object*); @@ -159,7 +158,7 @@ LEAN_EXPORT lean_object* l_Lean_isInductive___at___private_Lean_Elab_Tactic_Indu uint8_t l_Lean_LocalDecl_hasValue(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getAltNumFields___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_fvarId_x21(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalAlt___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalAlt___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalInduction___lambda__5(lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_environment_find(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_withAltsOfOptInductionAlts(lean_object*); @@ -168,7 +167,6 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tacti lean_object* l_Lean_MVarId_setKind(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getAltRHS(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalInduction___spec__3___lambda__1___boxed(lean_object*, lean_object*); lean_object* l_Lean_addBuiltinDeclarationRanges(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___lambda__4___boxed(lean_object**); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalInduction___lambda__5___boxed(lean_object**); @@ -186,9 +184,9 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_ElimApp_ uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_expandMultiAlt_x3f(lean_object*); +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__10; LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_withAltsOfOptInductionAlts___rarg___lambda__1___boxed(lean_object*); lean_object* l_Lean_stringToMessageData(lean_object*); -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__8; lean_object* l_Lean_Expr_mvar___override(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_setMotiveArg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -199,14 +197,15 @@ lean_object* l_Lean_Elab_Tactic_getFVarIds(lean_object*, lean_object*, lean_obje lean_object* l_Lean_RBNode_findCore___at_Lean_Meta_mkGeneralizationForbiddenSet_visit___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___lambda__8___boxed(lean_object**); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getArgExpectedType___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_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalInduction___spec__2___lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getNumExplicitFields___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_ElimApp_setMotiveArg___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalInduction__1___closed__5; LEAN_EXPORT lean_object* l_Array_zipWithAux___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_panic___at_Lean_Elab_Tactic_elabCasesTargets___spec__3___closed__1; lean_object* l_Lean_Meta_appendTag(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__12; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_expandInductionAlts_x3f___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_generalizeTargets(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalInduction___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutTacticIncrementality___at_Lean_Elab_Tactic_ElimApp_evalAlts_applyPreTac___spec__1(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -223,7 +222,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tac LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___spec__6(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalCases___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_altHasExplicitModifier(lean_object*); -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__7; LEAN_EXPORT uint8_t l_Lean_Elab_Tactic_isHoleRHS(lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___spec__5___at_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___lambda__3___closed__7; @@ -234,7 +232,6 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_ElimApp_ static lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getAltName___closed__5; static lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___lambda__1___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_hasMVar(lean_object*); @@ -276,7 +273,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_withReuseContext___at___private_Lean_E 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*); static lean_object* l_Lean_Elab_Tactic_ElimApp_instInhabitedAlt___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalCases__1___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_generalizeTargets___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_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getOptPreTacOfOptInductionAlts___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_tactic_customEliminators; @@ -295,13 +291,13 @@ static lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_g static lean_object* l_Lean_Elab_withSaveInfoContext___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___spec__2___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalInduction_checkTargets___spec__1___at_Lean_Elab_Tactic_evalInduction_checkTargets___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts___boxed(lean_object**); -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__3; LEAN_EXPORT lean_object* l_Lean_isInductive___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getNumExplicitFields(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_ElimApp_mkElimApp___closed__1; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_ElimApp_mkElimApp_loop___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_zip___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalAlt___spec__1___closed__1; +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__13; static lean_object* l_Lean_Elab_Term_withoutTacticIncrementality___at_Lean_Elab_Tactic_ElimApp_evalAlts_applyPreTac___spec__1___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___spec__3___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_elabTermForElim___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -319,6 +315,7 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalInduct LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getAltRHS___boxed(lean_object*); static lean_object* l_Lean_Elab_Tactic_ElimApp_setMotiveArg___closed__1; lean_object* l_Lean_registerTraceClass(lean_object*, uint8_t, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__7; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithIncremental___spec__7___lambda__2___boxed__const__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_SavedState_restore(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -342,6 +339,7 @@ LEAN_EXPORT uint8_t l_Std_Range_forIn_x27_loop___at_Lean_Elab_Tactic_ElimApp_eva lean_object* l_Lean_MessageData_ofFormat(lean_object*); lean_object* l_Lean_PersistentArray_append___rarg(lean_object*, lean_object*); lean_object* l_Lean_Elab_getBetterRef(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__11; lean_object* l_Lean_MVarId_withContext___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_synthPendingImp___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getAltVars(lean_object*); @@ -367,6 +365,8 @@ lean_object* l_Lean_log___at_Lean_Elab_Tactic_closeUsingOrAdmit___spec__3(lean_o LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___spec__1(lean_object*, lean_object*); lean_object* l_Lean_Elab_addBuiltinIncrementalElab(lean_object*, lean_object*); uint8_t l_List_isEmpty___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalInduction___spec__2___lambda__1(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__4; lean_object* lean_st_mk_ref(lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_synthesizeInstMVarCore(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_to_list(lean_object*); @@ -379,12 +379,14 @@ static lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___lambda__3__ lean_object* l_Lean_MVarId_withContext___at_Lean_Elab_Tactic_withMainContext___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_elabTermEnsuringType(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___lambda__8___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withReuseContext___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_withAltsOfOptInductionAlts___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_ElimApp_mkElimApp___spec__3(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithIncremental___spec__4___lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalAlt(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_levelZero; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161_(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_withAltsOfOptInductionAlts___rarg___lambda__1(lean_object*); lean_object* l_Lean_MVarId_revert(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_instInhabitedExpr; @@ -398,10 +400,11 @@ static lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_E LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalCases___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_ElimApp_mkElimApp___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabCasesTargets___boxed__const__1; -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__9; +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__9; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalInduction_declRange__1___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_generalizeTargets___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Tactic_getMainTarget___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__5; lean_object* l_List_lengthTRAux___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___lambda__6___closed__1; lean_object* l_Lean_Syntax_getSepArgs(lean_object*); @@ -412,9 +415,9 @@ LEAN_EXPORT lean_object* l_Array_zipWithAux___at_Lean_Elab_Tactic_ElimApp_evalAl LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithIncremental___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_name_eq(lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithIncremental___spec__4___closed__2; -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__4; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalInduction__1___closed__1; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withReuseContext___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_withAltsOfOptInductionAlts___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_addConstInfo___at_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_generalizeVars___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -450,6 +453,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalInduction_checkTargets___boxed(l LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_eraseIdx___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getAltLhses___boxed(lean_object*); static lean_object* l_Lean_Elab_Tactic_ElimApp_mkElimApp_loop___closed__2; extern lean_object* l_Std_Format_defWidth; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalCases_declRange__1___closed__4; @@ -461,7 +465,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSa LEAN_EXPORT lean_object* l_Lean_Elab_withSaveInfoContext___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getAltNumFields___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_instInhabitedMetaM___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__2; extern lean_object* l_Lean_instInhabitedFVarId; static lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___lambda__3___closed__1; static lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_generalizeTargets___closed__1; @@ -485,6 +488,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalInduction___lambda__3(lean_objec lean_object* l_Lean_Elab_Term_ensureHasType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalInduction_declRange__1___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithIncremental___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__5; lean_object* l_Lean_Name_mkStr6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getUserGeneralizingFVarIds___closed__1; lean_object* l_Lean_Elab_Tactic_saveState___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -496,11 +500,12 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tac LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_closeUsingOrAdmit(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabCasesTargets___lambda__2(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__6; +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__3; lean_object* l_Lean_Syntax_setArg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_mkElimApp_loop___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_introNCore(lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getAltName___closed__7; -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__5; LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__1(lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalInduction_checkTargets___spec__1___at_Lean_Elab_Tactic_evalInduction_checkTargets___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -530,19 +535,20 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalInduction___lambda__2(lean_objec LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getArgExpectedType___boxed(lean_object*); lean_object* l_Lean_Expr_app___override(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalCases__1___closed__3; +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__15; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___lambda__6___boxed(lean_object**); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalInduction_checkTargets___spec__1(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); lean_object* l_Lean_MVarId_getDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalInduction__2(lean_object*); lean_object* l_Lean_Elab_getResetInfoTrees___at_Lean_Elab_Term_withDeclName___spec__3___rarg(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__11; LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getAltDArrow(lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getUserGeneralizingFVarIds___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getOptPreTacOfOptInductionAlts(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_generalizeVars___spec__1___lambda__2___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___spec__13(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__4; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_checkAltsOfOptInductionAlts___spec__1(lean_object*, size_t, size_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapM___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalInduction_checkTargets___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -574,6 +580,7 @@ lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMe LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalInduction___lambda__4___boxed(lean_object**); lean_object* l_Lean_isTracingEnabledFor___at_Lean_Elab_Tactic_evalTactic_handleEx___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalCases__1___closed__4; +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__2; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_ElimApp_mkElimApp___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_isNone(lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -583,12 +590,12 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tacti LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___lambda__2(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___boxed__const__1; static lean_object* l_Lean_Elab_Tactic_evalAlt___lambda__3___closed__1; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalInduction___spec__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalAlt___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_nat_sub(lean_object*, lean_object*); lean_object* l_Lean_MVarId_tryClear(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_getAppFn(lean_object*); static lean_object* l_Lean_Elab_Tactic_elabCasesTargets___lambda__1___closed__1; +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__8; LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getOptPreTacOfOptInductionAlts___boxed(lean_object*); lean_object* l_Lean_Syntax_getRange_x3f(lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts___lambda__1___boxed(lean_object**); @@ -605,10 +612,8 @@ lean_object* l_Lean_RBNode_insert___at_Lean_FVarIdSet_insert___spec__1(lean_obje static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalCases_declRange__1___closed__5; static lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithIncremental___spec__4___closed__3; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Tactic_elabCasesTargets___spec__5(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__13; lean_object* lean_erase_macro_scopes(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getBindingName___boxed(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalInduction___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_reverse___rarg(lean_object*); static lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getAltName___closed__2; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_checkAltsOfOptInductionAlts___spec__1___lambda__2___closed__3; @@ -621,17 +626,16 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_withReuseContext___at___private_Lean_E LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getFType___boxed(lean_object*); static lean_object* l_Lean_Elab_Term_withoutTacticIncrementality___at_Lean_Elab_Tactic_ElimApp_evalAlts_applyPreTac___spec__1___closed__5; uint8_t l_Lean_Syntax_hasMissing(lean_object*); -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__15; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutTacticIncrementality___at_Lean_Elab_Tactic_ElimApp_evalAlts_applyPreTac___spec__1___lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___boxed(lean_object**); size_t lean_usize_add(size_t, size_t); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_checkAltsOfOptInductionAlts___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalInduction___lambda__3___boxed(lean_object**); -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__14; static lean_object* l_Lean_Elab_Tactic_ElimApp_mkElimApp_loop___closed__4; -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__16; static lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___lambda__8___closed__7; static lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___lambda__6___closed__4; +lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalGeneralize___spec__9(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_withAltsOfOptInductionAlts___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___lambda__3___closed__1; 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*); @@ -668,27 +672,26 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutTacticIncrementality___at_Lean_ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithIncremental___spec__7___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_withTacticInfoContext___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalInduction_declRange__1___closed__7; -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__4; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithIncremental___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_string_append(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_withSaveInfoContext___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalInduction_checkTargets(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__6; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalCases__2(lean_object*); lean_object* l_Lean_Meta_mkFreshExprSyntheticOpaqueMVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_shouldGeneralizeTarget___boxed(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_getFirstAltLhs___boxed(lean_object*); lean_object* lean_array_get_size(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalInduction___spec__2(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___spec__11(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_generalizeTargets___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_Std_Range_forIn_x27_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_isHoleRHS___boxed(lean_object*); static lean_object* l_Lean_Elab_Tactic_getInductiveValFromMajor___lambda__1___closed__2; lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getNumExplicitFields___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103_(lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); uint8_t l_Array_contains___at___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps_visit___spec__2(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_withAltsOfOptInductionAlts___rarg___lambda__1___closed__2; @@ -708,18 +711,17 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_ElimApp_mkElimA lean_object* l_Lean_mkConstWithLevelParams___at_Lean_Elab_Term_expandDeclId___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___lambda__3___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___lambda__1___boxed(lean_object**); -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__5; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_ElimApp_mkElimApp___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Term_withNarrowedTacticReuse___at_Lean_Elab_Tactic_evalInduction___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isFVar(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___spec__7(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_mvarId_x21(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalCases___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___lambda__5___closed__2; -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__2; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalInduction_checkTargets___spec__1___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithIncremental___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_getResetInfoTrees___at_Lean_Elab_Tactic_withTacticInfoContext___spec__2___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getAltLhses(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalInduction_declRange__1___closed__5; static lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getAltNumFields___lambda__1___closed__2; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); @@ -747,6 +749,24 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalAlt___lambda__4(lean_object*, le LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getFType___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___lambda__3___boxed(lean_object**); uint8_t l_Array_isEmpty___rarg(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getAltLhses(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; +x_2 = lean_unsigned_to_nat(0u); +x_3 = l_Lean_Syntax_getArg(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getAltLhses___boxed(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getAltLhses(x_1); +lean_dec(x_1); +return x_2; +} +} LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getFirstAltLhs(lean_object* x_1) { _start: { @@ -1216,31 +1236,51 @@ return x_18; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalAlt___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalAlt___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { -lean_object* x_14; uint8_t x_15; -x_14 = l_Lean_Elab_Tactic_getGoals___rarg(x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -x_15 = !lean_is_exclusive(x_14); -if (x_15 == 0) +lean_object* x_15; uint8_t x_16; +x_15 = l_Lean_Elab_Tactic_getGoals___rarg(x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +x_16 = !lean_is_exclusive(x_15); +if (x_16 == 0) { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_16 = lean_ctor_get(x_14, 0); -x_17 = lean_ctor_get(x_14, 1); -x_18 = lean_box(0); -lean_ctor_set_tag(x_14, 1); -lean_ctor_set(x_14, 1, x_18); -lean_ctor_set(x_14, 0, x_1); -x_19 = l_Lean_Elab_Tactic_setGoals(x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_17); -x_20 = lean_ctor_get(x_19, 1); -lean_inc(x_20); -lean_dec(x_19); -x_21 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalAlt___lambda__1), 11, 2); -lean_closure_set(x_21, 0, x_2); -lean_closure_set(x_21, 1, x_3); -x_22 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); -lean_closure_set(x_22, 0, x_4); -lean_closure_set(x_22, 1, x_21); +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_17 = lean_ctor_get(x_15, 0); +x_18 = lean_ctor_get(x_15, 1); +x_19 = lean_box(0); +lean_ctor_set_tag(x_15, 1); +lean_ctor_set(x_15, 1, x_19); +lean_ctor_set(x_15, 0, x_1); +x_20 = l_Lean_Elab_Tactic_setGoals(x_15, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_18); +x_21 = !lean_is_exclusive(x_20); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_22 = lean_ctor_get(x_20, 1); +x_23 = lean_ctor_get(x_20, 0); +lean_dec(x_23); +x_24 = lean_unsigned_to_nat(0u); +x_25 = l_Lean_Syntax_getArg(x_2, x_24); +lean_ctor_set_tag(x_20, 1); +lean_ctor_set(x_20, 1, x_19); +lean_ctor_set(x_20, 0, x_3); +x_26 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_20); +x_27 = lean_array_mk(x_26); +x_28 = lean_box(2); +x_29 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalAlt___spec__1___closed__2; +x_30 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +lean_ctor_set(x_30, 2, x_27); +x_31 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalAlt___lambda__1), 11, 2); +lean_closure_set(x_31, 0, x_4); +lean_closure_set(x_31, 1, x_5); +x_32 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); +lean_closure_set(x_32, 0, x_30); +lean_closure_set(x_32, 1, x_31); +lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); @@ -1248,17 +1288,17 @@ lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -lean_inc(x_5); -x_23 = l_Lean_Elab_Tactic_closeUsingOrAdmit(x_22, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_20); -if (lean_obj_tag(x_23) == 0) +x_33 = l_Lean_Elab_Tactic_closeUsingOrAdmit(x_32, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_22); +if (lean_obj_tag(x_33) == 0) { -lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_23, 1); -lean_inc(x_25); -lean_dec(x_23); -x_26 = l_Lean_Elab_Tactic_setGoals(x_16, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_25); +lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; +x_34 = lean_ctor_get(x_33, 0); +lean_inc(x_34); +x_35 = lean_ctor_get(x_33, 1); +lean_inc(x_35); +lean_dec(x_33); +x_36 = l_Lean_Elab_Tactic_setGoals(x_17, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_35); +lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -1266,37 +1306,37 @@ lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -x_27 = !lean_is_exclusive(x_26); -if (x_27 == 0) +x_37 = !lean_is_exclusive(x_36); +if (x_37 == 0) { -lean_object* x_28; -x_28 = lean_ctor_get(x_26, 0); -lean_dec(x_28); -lean_ctor_set(x_26, 0, x_24); -return x_26; +lean_object* x_38; +x_38 = lean_ctor_get(x_36, 0); +lean_dec(x_38); +lean_ctor_set(x_36, 0, x_34); +return x_36; } else { -lean_object* x_29; lean_object* x_30; -x_29 = lean_ctor_get(x_26, 1); -lean_inc(x_29); -lean_dec(x_26); -x_30 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_30, 0, x_24); -lean_ctor_set(x_30, 1, x_29); -return x_30; +lean_object* x_39; lean_object* x_40; +x_39 = lean_ctor_get(x_36, 1); +lean_inc(x_39); +lean_dec(x_36); +x_40 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_40, 0, x_34); +lean_ctor_set(x_40, 1, x_39); +return x_40; } } else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; -x_31 = lean_ctor_get(x_23, 0); -lean_inc(x_31); -x_32 = lean_ctor_get(x_23, 1); -lean_inc(x_32); -lean_dec(x_23); -x_33 = l_Lean_Elab_Tactic_setGoals(x_16, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_32); +lean_object* x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; +x_41 = lean_ctor_get(x_33, 0); +lean_inc(x_41); +x_42 = lean_ctor_get(x_33, 1); +lean_inc(x_42); +lean_dec(x_33); +x_43 = l_Lean_Elab_Tactic_setGoals(x_17, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_42); +lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -1304,52 +1344,57 @@ lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -x_34 = !lean_is_exclusive(x_33); -if (x_34 == 0) +x_44 = !lean_is_exclusive(x_43); +if (x_44 == 0) { -lean_object* x_35; -x_35 = lean_ctor_get(x_33, 0); -lean_dec(x_35); -lean_ctor_set_tag(x_33, 1); -lean_ctor_set(x_33, 0, x_31); -return x_33; +lean_object* x_45; +x_45 = lean_ctor_get(x_43, 0); +lean_dec(x_45); +lean_ctor_set_tag(x_43, 1); +lean_ctor_set(x_43, 0, x_41); +return x_43; } else { -lean_object* x_36; lean_object* x_37; -x_36 = lean_ctor_get(x_33, 1); -lean_inc(x_36); -lean_dec(x_33); -x_37 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_37, 0, x_31); -lean_ctor_set(x_37, 1, x_36); -return x_37; +lean_object* x_46; lean_object* x_47; +x_46 = lean_ctor_get(x_43, 1); +lean_inc(x_46); +lean_dec(x_43); +x_47 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_47, 0, x_41); +lean_ctor_set(x_47, 1, x_46); +return x_47; } } } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_38 = lean_ctor_get(x_14, 0); -x_39 = lean_ctor_get(x_14, 1); -lean_inc(x_39); -lean_inc(x_38); -lean_dec(x_14); -x_40 = lean_box(0); -x_41 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_41, 0, x_1); -lean_ctor_set(x_41, 1, x_40); -x_42 = l_Lean_Elab_Tactic_setGoals(x_41, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_39); -x_43 = lean_ctor_get(x_42, 1); -lean_inc(x_43); -lean_dec(x_42); -x_44 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalAlt___lambda__1), 11, 2); -lean_closure_set(x_44, 0, x_2); -lean_closure_set(x_44, 1, x_3); -x_45 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); -lean_closure_set(x_45, 0, x_4); -lean_closure_set(x_45, 1, x_44); +lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_48 = lean_ctor_get(x_20, 1); +lean_inc(x_48); +lean_dec(x_20); +x_49 = lean_unsigned_to_nat(0u); +x_50 = l_Lean_Syntax_getArg(x_2, x_49); +x_51 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_51, 0, x_3); +lean_ctor_set(x_51, 1, x_19); +x_52 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_52, 0, x_50); +lean_ctor_set(x_52, 1, x_51); +x_53 = lean_array_mk(x_52); +x_54 = lean_box(2); +x_55 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalAlt___spec__1___closed__2; +x_56 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_56, 0, x_54); +lean_ctor_set(x_56, 1, x_55); +lean_ctor_set(x_56, 2, x_53); +x_57 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalAlt___lambda__1), 11, 2); +lean_closure_set(x_57, 0, x_4); +lean_closure_set(x_57, 1, x_5); +x_58 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); +lean_closure_set(x_58, 0, x_56); +lean_closure_set(x_58, 1, x_57); +lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); @@ -1357,17 +1402,17 @@ lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -lean_inc(x_5); -x_46 = l_Lean_Elab_Tactic_closeUsingOrAdmit(x_45, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_43); -if (lean_obj_tag(x_46) == 0) +x_59 = l_Lean_Elab_Tactic_closeUsingOrAdmit(x_58, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_48); +if (lean_obj_tag(x_59) == 0) { -lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_47 = lean_ctor_get(x_46, 0); -lean_inc(x_47); -x_48 = lean_ctor_get(x_46, 1); -lean_inc(x_48); -lean_dec(x_46); -x_49 = l_Lean_Elab_Tactic_setGoals(x_38, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_48); +lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_60 = lean_ctor_get(x_59, 0); +lean_inc(x_60); +x_61 = lean_ctor_get(x_59, 1); +lean_inc(x_61); +lean_dec(x_59); +x_62 = l_Lean_Elab_Tactic_setGoals(x_17, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_61); +lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -1375,35 +1420,35 @@ lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -x_50 = lean_ctor_get(x_49, 1); -lean_inc(x_50); -if (lean_is_exclusive(x_49)) { - lean_ctor_release(x_49, 0); - lean_ctor_release(x_49, 1); - x_51 = x_49; +x_63 = lean_ctor_get(x_62, 1); +lean_inc(x_63); +if (lean_is_exclusive(x_62)) { + lean_ctor_release(x_62, 0); + lean_ctor_release(x_62, 1); + x_64 = x_62; } else { - lean_dec_ref(x_49); - x_51 = lean_box(0); + lean_dec_ref(x_62); + x_64 = lean_box(0); } -if (lean_is_scalar(x_51)) { - x_52 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_64)) { + x_65 = lean_alloc_ctor(0, 2, 0); } else { - x_52 = x_51; + x_65 = x_64; } -lean_ctor_set(x_52, 0, x_47); -lean_ctor_set(x_52, 1, x_50); -return x_52; +lean_ctor_set(x_65, 0, x_60); +lean_ctor_set(x_65, 1, x_63); +return x_65; } else { -lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; -x_53 = lean_ctor_get(x_46, 0); -lean_inc(x_53); -x_54 = lean_ctor_get(x_46, 1); -lean_inc(x_54); -lean_dec(x_46); -x_55 = l_Lean_Elab_Tactic_setGoals(x_38, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_54); +lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; +x_66 = lean_ctor_get(x_59, 0); +lean_inc(x_66); +x_67 = lean_ctor_get(x_59, 1); +lean_inc(x_67); +lean_dec(x_59); +x_68 = l_Lean_Elab_Tactic_setGoals(x_17, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_67); +lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -1411,26 +1456,158 @@ lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -x_56 = lean_ctor_get(x_55, 1); -lean_inc(x_56); -if (lean_is_exclusive(x_55)) { - lean_ctor_release(x_55, 0); - lean_ctor_release(x_55, 1); - x_57 = x_55; +x_69 = lean_ctor_get(x_68, 1); +lean_inc(x_69); +if (lean_is_exclusive(x_68)) { + lean_ctor_release(x_68, 0); + lean_ctor_release(x_68, 1); + x_70 = x_68; } else { - lean_dec_ref(x_55); - x_57 = lean_box(0); + lean_dec_ref(x_68); + x_70 = lean_box(0); } -if (lean_is_scalar(x_57)) { - x_58 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_70)) { + x_71 = lean_alloc_ctor(1, 2, 0); } else { - x_58 = x_57; - lean_ctor_set_tag(x_58, 1); + x_71 = x_70; + lean_ctor_set_tag(x_71, 1); } -lean_ctor_set(x_58, 0, x_53); -lean_ctor_set(x_58, 1, x_56); -return x_58; +lean_ctor_set(x_71, 0, x_66); +lean_ctor_set(x_71, 1, x_69); +return x_71; +} +} +} +else +{ +lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; +x_72 = lean_ctor_get(x_15, 0); +x_73 = lean_ctor_get(x_15, 1); +lean_inc(x_73); +lean_inc(x_72); +lean_dec(x_15); +x_74 = lean_box(0); +x_75 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_75, 0, x_1); +lean_ctor_set(x_75, 1, x_74); +x_76 = l_Lean_Elab_Tactic_setGoals(x_75, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_73); +x_77 = lean_ctor_get(x_76, 1); +lean_inc(x_77); +if (lean_is_exclusive(x_76)) { + lean_ctor_release(x_76, 0); + lean_ctor_release(x_76, 1); + x_78 = x_76; +} else { + lean_dec_ref(x_76); + x_78 = lean_box(0); +} +x_79 = lean_unsigned_to_nat(0u); +x_80 = l_Lean_Syntax_getArg(x_2, x_79); +if (lean_is_scalar(x_78)) { + x_81 = lean_alloc_ctor(1, 2, 0); +} else { + x_81 = x_78; + lean_ctor_set_tag(x_81, 1); +} +lean_ctor_set(x_81, 0, x_3); +lean_ctor_set(x_81, 1, x_74); +x_82 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_82, 0, x_80); +lean_ctor_set(x_82, 1, x_81); +x_83 = lean_array_mk(x_82); +x_84 = lean_box(2); +x_85 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalAlt___spec__1___closed__2; +x_86 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_86, 0, x_84); +lean_ctor_set(x_86, 1, x_85); +lean_ctor_set(x_86, 2, x_83); +x_87 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalAlt___lambda__1), 11, 2); +lean_closure_set(x_87, 0, x_4); +lean_closure_set(x_87, 1, x_5); +x_88 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); +lean_closure_set(x_88, 0, x_86); +lean_closure_set(x_88, 1, x_87); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +x_89 = l_Lean_Elab_Tactic_closeUsingOrAdmit(x_88, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_77); +if (lean_obj_tag(x_89) == 0) +{ +lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; +x_90 = lean_ctor_get(x_89, 0); +lean_inc(x_90); +x_91 = lean_ctor_get(x_89, 1); +lean_inc(x_91); +lean_dec(x_89); +x_92 = l_Lean_Elab_Tactic_setGoals(x_72, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_91); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +x_93 = lean_ctor_get(x_92, 1); +lean_inc(x_93); +if (lean_is_exclusive(x_92)) { + lean_ctor_release(x_92, 0); + lean_ctor_release(x_92, 1); + x_94 = x_92; +} else { + lean_dec_ref(x_92); + x_94 = lean_box(0); +} +if (lean_is_scalar(x_94)) { + x_95 = lean_alloc_ctor(0, 2, 0); +} else { + x_95 = x_94; +} +lean_ctor_set(x_95, 0, x_90); +lean_ctor_set(x_95, 1, x_93); +return x_95; +} +else +{ +lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; +x_96 = lean_ctor_get(x_89, 0); +lean_inc(x_96); +x_97 = lean_ctor_get(x_89, 1); +lean_inc(x_97); +lean_dec(x_89); +x_98 = l_Lean_Elab_Tactic_setGoals(x_72, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_97); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +x_99 = lean_ctor_get(x_98, 1); +lean_inc(x_99); +if (lean_is_exclusive(x_98)) { + lean_ctor_release(x_98, 0); + lean_ctor_release(x_98, 1); + x_100 = x_98; +} else { + lean_dec_ref(x_98); + x_100 = lean_box(0); +} +if (lean_is_scalar(x_100)) { + x_101 = lean_alloc_ctor(1, 2, 0); +} else { + x_101 = x_100; + lean_ctor_set_tag(x_101, 1); +} +lean_ctor_set(x_101, 0, x_96); +lean_ctor_set(x_101, 1, x_99); +return x_101; } } } @@ -1671,11 +1848,13 @@ if (x_17 == 0) { lean_object* x_18; lean_object* x_19; lean_inc(x_14); -x_18 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalAlt___lambda__2), 13, 4); +lean_inc(x_16); +x_18 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalAlt___lambda__2___boxed), 14, 5); lean_closure_set(x_18, 0, x_1); -lean_closure_set(x_18, 1, x_3); -lean_closure_set(x_18, 2, x_14); -lean_closure_set(x_18, 3, x_2); +lean_closure_set(x_18, 1, x_2); +lean_closure_set(x_18, 2, x_16); +lean_closure_set(x_18, 3, x_3); +lean_closure_set(x_18, 4, x_14); x_19 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalAlt___spec__1(x_16, x_14, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); return x_19; } @@ -1693,6 +1872,15 @@ return x_21; } } } +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalAlt___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; +x_15 = l_Lean_Elab_Tactic_evalAlt___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_2); +return x_15; +} +} static lean_object* _init_l_Lean_Elab_Tactic_ElimApp_instInhabitedAlt___closed__1() { _start: { @@ -16186,7 +16374,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; uint8_t x_9; @@ -16775,7 +16963,7 @@ lean_inc(x_35); lean_dec(x_34); x_36 = lean_array_get_size(x_11); x_37 = lean_mk_empty_array_with_capacity(x_36); -x_38 = l_Array_mapIdxM_map___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___spec__2(x_3, x_11, x_11, x_36, x_27, lean_box(0), x_37); +x_38 = l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___spec__2(x_3, x_11, x_11, x_36, x_27, lean_box(0), x_37); lean_inc(x_19); lean_inc(x_18); lean_inc(x_17); @@ -17034,11 +17222,11 @@ lean_dec(x_1); return x_5; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; -x_8 = l_Array_mapIdxM_map___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_3); lean_dec(x_2); return x_8; @@ -21775,7 +21963,7 @@ lean_dec(x_2); return x_10; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__1() { _start: { lean_object* x_1; @@ -21783,7 +21971,7 @@ x_1 = lean_mk_string_unchecked("tactic", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__2() { _start: { lean_object* x_1; @@ -21791,17 +21979,17 @@ x_1 = lean_mk_string_unchecked("customEliminators", 17, 17); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__1; -x_2 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__2; +x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__1; +x_2 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__2; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__4() { _start: { lean_object* x_1; @@ -21809,13 +21997,13 @@ x_1 = lean_mk_string_unchecked("enable using custom eliminators in the 'inductio return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__5() { _start: { uint8_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = 1; -x_2 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__1; -x_3 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__4; +x_2 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__1; +x_3 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__4; x_4 = lean_box(x_1); x_5 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_5, 0, x_4); @@ -21824,26 +22012,26 @@ lean_ctor_set(x_5, 2, x_3); return x_5; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__6() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getAltName___closed__1; x_2 = l_Lean_Elab_Term_withoutTacticIncrementality___at_Lean_Elab_Tactic_ElimApp_evalAlts_applyPreTac___spec__1___closed__2; x_3 = l_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___lambda__3___closed__1; -x_4 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__1; -x_5 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__2; +x_4 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__1; +x_5 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__2; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_2 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__3; -x_3 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__5; -x_4 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__6; +x_2 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__3; +x_3 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__5; +x_4 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__6; x_5 = l_Lean_Option_register___at_Lean_Elab_initFn____x40_Lean_Elab_AutoBound___hyg_6____spec__1(x_2, x_3, x_4, x_1); return x_5; } @@ -24024,33 +24212,7 @@ return x_30; } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalInduction___spec__2(size_t x_1, size_t x_2, lean_object* x_3) { -_start: -{ -uint8_t x_4; -x_4 = lean_usize_dec_lt(x_2, x_1); -if (x_4 == 0) -{ -return x_3; -} -else -{ -lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; size_t x_9; size_t x_10; lean_object* x_11; -x_5 = lean_array_uget(x_3, x_2); -x_6 = lean_unsigned_to_nat(0u); -x_7 = lean_array_uset(x_3, x_2, x_6); -x_8 = l_Lean_Expr_fvarId_x21(x_5); -lean_dec(x_5); -x_9 = 1; -x_10 = lean_usize_add(x_2, x_9); -x_11 = lean_array_uset(x_7, x_2, x_8); -x_2 = x_10; -x_3 = x_11; -goto _start; -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___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_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___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) { _start: { uint8_t x_12; @@ -24183,7 +24345,7 @@ return x_50; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_withNarrowedTacticReuse___at_Lean_Elab_Tactic_evalInduction___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_EXPORT lean_object* l_Lean_Elab_Term_withNarrowedTacticReuse___at_Lean_Elab_Tactic_evalInduction___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; @@ -24214,7 +24376,7 @@ x_20 = lean_ctor_get(x_6, 8); lean_dec(x_20); x_21 = lean_box(0); lean_ctor_set(x_6, 8, x_21); -x_22 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__5(x_15, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_22 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__4(x_15, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); return x_22; } else @@ -24268,7 +24430,7 @@ lean_ctor_set_uint8(x_42, sizeof(void*)*9 + 6, x_36); lean_ctor_set_uint8(x_42, sizeof(void*)*9 + 7, x_37); lean_ctor_set_uint8(x_42, sizeof(void*)*9 + 8, x_39); lean_ctor_set_uint8(x_42, sizeof(void*)*9 + 9, x_40); -x_43 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__5(x_15, x_17, x_4, x_5, x_42, x_7, x_8, x_9, x_10, x_11, x_12); +x_43 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__4(x_15, x_17, x_4, x_5, x_42, x_7, x_8, x_9, x_10, x_11, x_12); return x_43; } } @@ -24302,7 +24464,7 @@ x_50 = lean_ctor_get(x_45, 0); lean_dec(x_50); x_51 = lean_box(0); lean_ctor_set(x_45, 0, x_51); -x_52 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__5(x_15, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_52 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__4(x_15, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); return x_52; } else @@ -24316,7 +24478,7 @@ x_55 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_55, 0, x_54); lean_ctor_set(x_55, 1, x_53); lean_ctor_set(x_18, 0, x_55); -x_56 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__5(x_15, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_56 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__4(x_15, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); return x_56; } } @@ -24389,7 +24551,7 @@ lean_ctor_set_uint8(x_79, sizeof(void*)*9 + 6, x_70); lean_ctor_set_uint8(x_79, sizeof(void*)*9 + 7, x_71); lean_ctor_set_uint8(x_79, sizeof(void*)*9 + 8, x_73); lean_ctor_set_uint8(x_79, sizeof(void*)*9 + 9, x_74); -x_80 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__5(x_15, x_17, x_4, x_5, x_79, x_7, x_8, x_9, x_10, x_11, x_12); +x_80 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__4(x_15, x_17, x_4, x_5, x_79, x_7, x_8, x_9, x_10, x_11, x_12); return x_80; } } @@ -24440,14 +24602,14 @@ x_95 = lean_box(0); lean_ctor_set(x_45, 0, x_95); lean_ctor_set(x_46, 0, x_45); lean_ctor_set(x_6, 8, x_46); -x_96 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__5(x_15, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_96 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__4(x_15, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); return x_96; } else { lean_object* x_97; lean_ctor_set(x_83, 0, x_92); -x_97 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__5(x_15, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_97 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__4(x_15, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); return x_97; } } @@ -24479,7 +24641,7 @@ x_105 = lean_box(0); lean_ctor_set(x_45, 0, x_105); lean_ctor_set(x_46, 0, x_45); lean_ctor_set(x_6, 8, x_46); -x_106 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__5(x_15, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_106 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__4(x_15, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); return x_106; } else @@ -24489,7 +24651,7 @@ x_107 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_107, 0, x_102); lean_ctor_set(x_107, 1, x_99); lean_ctor_set(x_46, 0, x_107); -x_108 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__5(x_15, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_108 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__4(x_15, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); return x_108; } } @@ -24535,7 +24697,7 @@ lean_ctor_set(x_119, 0, x_118); lean_ctor_set(x_119, 1, x_109); lean_ctor_set(x_46, 0, x_119); lean_ctor_set(x_6, 8, x_46); -x_120 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__5(x_15, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_120 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__4(x_15, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); return x_120; } else @@ -24553,7 +24715,7 @@ x_122 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_122, 0, x_46); lean_ctor_set(x_122, 1, x_109); lean_ctor_set(x_18, 0, x_122); -x_123 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__5(x_15, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_123 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__4(x_15, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); return x_123; } } @@ -24657,7 +24819,7 @@ lean_ctor_set_uint8(x_155, sizeof(void*)*9 + 6, x_138); lean_ctor_set_uint8(x_155, sizeof(void*)*9 + 7, x_139); lean_ctor_set_uint8(x_155, sizeof(void*)*9 + 8, x_141); lean_ctor_set_uint8(x_155, sizeof(void*)*9 + 9, x_142); -x_156 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__5(x_15, x_17, x_4, x_5, x_155, x_7, x_8, x_9, x_10, x_11, x_12); +x_156 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__4(x_15, x_17, x_4, x_5, x_155, x_7, x_8, x_9, x_10, x_11, x_12); return x_156; } else @@ -24699,7 +24861,7 @@ lean_ctor_set_uint8(x_159, sizeof(void*)*9 + 6, x_138); lean_ctor_set_uint8(x_159, sizeof(void*)*9 + 7, x_139); lean_ctor_set_uint8(x_159, sizeof(void*)*9 + 8, x_141); lean_ctor_set_uint8(x_159, sizeof(void*)*9 + 9, x_142); -x_160 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__5(x_15, x_17, x_4, x_5, x_159, x_7, x_8, x_9, x_10, x_11, x_12); +x_160 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__4(x_15, x_17, x_4, x_5, x_159, x_7, x_8, x_9, x_10, x_11, x_12); return x_160; } } @@ -24824,7 +24986,7 @@ lean_ctor_set_uint8(x_194, sizeof(void*)*9 + 6, x_175); lean_ctor_set_uint8(x_194, sizeof(void*)*9 + 7, x_176); lean_ctor_set_uint8(x_194, sizeof(void*)*9 + 8, x_178); lean_ctor_set_uint8(x_194, sizeof(void*)*9 + 9, x_179); -x_195 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__5(x_15, x_17, x_4, x_5, x_194, x_7, x_8, x_9, x_10, x_11, x_12); +x_195 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__4(x_15, x_17, x_4, x_5, x_194, x_7, x_8, x_9, x_10, x_11, x_12); return x_195; } else @@ -24871,7 +25033,7 @@ lean_ctor_set_uint8(x_199, sizeof(void*)*9 + 6, x_175); lean_ctor_set_uint8(x_199, sizeof(void*)*9 + 7, x_176); lean_ctor_set_uint8(x_199, sizeof(void*)*9 + 8, x_178); lean_ctor_set_uint8(x_199, sizeof(void*)*9 + 9, x_179); -x_200 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__5(x_15, x_17, x_4, x_5, x_199, x_7, x_8, x_9, x_10, x_11, x_12); +x_200 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__4(x_15, x_17, x_4, x_5, x_199, x_7, x_8, x_9, x_10, x_11, x_12); return x_200; } } @@ -24976,7 +25138,7 @@ lean_ctor_set_uint8(x_227, sizeof(void*)*9 + 6, x_216); lean_ctor_set_uint8(x_227, sizeof(void*)*9 + 7, x_217); lean_ctor_set_uint8(x_227, sizeof(void*)*9 + 8, x_219); lean_ctor_set_uint8(x_227, sizeof(void*)*9 + 9, x_220); -x_228 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__5(x_15, x_17, x_4, x_5, x_227, x_7, x_8, x_9, x_10, x_11, x_12); +x_228 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__4(x_15, x_17, x_4, x_5, x_227, x_7, x_8, x_9, x_10, x_11, x_12); return x_228; } else @@ -25108,7 +25270,7 @@ lean_ctor_set_uint8(x_263, sizeof(void*)*9 + 6, x_244); lean_ctor_set_uint8(x_263, sizeof(void*)*9 + 7, x_245); lean_ctor_set_uint8(x_263, sizeof(void*)*9 + 8, x_247); lean_ctor_set_uint8(x_263, sizeof(void*)*9 + 9, x_248); -x_264 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__5(x_15, x_17, x_4, x_5, x_263, x_7, x_8, x_9, x_10, x_11, x_12); +x_264 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__4(x_15, x_17, x_4, x_5, x_263, x_7, x_8, x_9, x_10, x_11, x_12); return x_264; } else @@ -25160,7 +25322,7 @@ lean_ctor_set_uint8(x_269, sizeof(void*)*9 + 6, x_244); lean_ctor_set_uint8(x_269, sizeof(void*)*9 + 7, x_245); lean_ctor_set_uint8(x_269, sizeof(void*)*9 + 8, x_247); lean_ctor_set_uint8(x_269, sizeof(void*)*9 + 9, x_248); -x_270 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__5(x_15, x_17, x_4, x_5, x_269, x_7, x_8, x_9, x_10, x_11, x_12); +x_270 = l_Lean_Elab_Term_withReuseContext___at_Lean_Elab_Tactic_evalInduction___spec__4(x_15, x_17, x_4, x_5, x_269, x_7, x_8, x_9, x_10, x_11, x_12); return x_270; } } @@ -25168,7 +25330,7 @@ return x_270; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalInduction___spec__3___lambda__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalInduction___spec__2___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; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; @@ -25192,13 +25354,13 @@ lean_ctor_set(x_11, 1, x_10); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalInduction___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalInduction___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; -x_13 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalInduction___spec__3___lambda__1___boxed), 2, 1); +x_13 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalInduction___spec__2___lambda__1___boxed), 2, 1); lean_closure_set(x_13, 0, x_1); -x_14 = l_Lean_Elab_Term_withNarrowedTacticReuse___at_Lean_Elab_Tactic_evalInduction___spec__4(x_13, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_14 = l_Lean_Elab_Term_withNarrowedTacticReuse___at_Lean_Elab_Tactic_evalInduction___spec__3(x_13, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); return x_14; } } @@ -25324,7 +25486,7 @@ lean_closure_set(x_21, 3, x_5); lean_closure_set(x_21, 4, x_6); lean_closure_set(x_21, 5, x_3); x_22 = lean_unsigned_to_nat(4u); -x_23 = l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalInduction___spec__3(x_22, x_21, x_7, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_20); +x_23 = l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalInduction___spec__2(x_22, x_21, x_7, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_20); return x_23; } else @@ -25586,7 +25748,7 @@ lean_inc(x_22); lean_dec(x_21); x_23 = lean_array_size(x_19); lean_inc(x_19); -x_24 = l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalInduction___spec__2(x_23, x_3, x_19); +x_24 = l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalGeneralize___spec__9(x_23, x_3, x_19); lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); @@ -26181,23 +26343,11 @@ x_15 = l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalInduction___spec__1(x_13 return x_15; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalInduction___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -size_t x_4; size_t x_5; lean_object* x_6; -x_4 = lean_unbox_usize(x_1); -lean_dec(x_1); -x_5 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_6 = l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalInduction___spec__2(x_4, x_5, x_3); -return x_6; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalInduction___spec__3___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalInduction___spec__2___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalInduction___spec__3___lambda__1(x_1, x_2); +x_3 = l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalInduction___spec__2___lambda__1(x_1, x_2); lean_dec(x_2); return x_3; } @@ -27306,7 +27456,7 @@ static lean_object* _init_l_Lean_Elab_Tactic_elabCasesTargets___lambda__1___clos lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Elab_Tactic_elabCasesTargets___lambda__1___closed__4; x_2 = l_Lean_Elab_Tactic_elabCasesTargets___lambda__1___closed__5; -x_3 = lean_unsigned_to_nat(713u); +x_3 = lean_unsigned_to_nat(717u); x_4 = lean_unsigned_to_nat(8u); x_5 = l_Lean_Elab_Tactic_elabCasesTargets___lambda__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -28657,7 +28807,7 @@ lean_closure_set(x_24, 3, x_8); lean_closure_set(x_24, 4, x_3); lean_closure_set(x_24, 5, x_9); x_25 = lean_unsigned_to_nat(3u); -x_26 = l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalInduction___spec__3(x_25, x_24, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_23); +x_26 = l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalInduction___spec__2(x_25, x_24, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_23); return x_26; } else @@ -29653,7 +29803,7 @@ x_3 = l_Lean_Elab_addBuiltinIncrementalElab(x_2, x_1); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -29663,7 +29813,7 @@ x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -29673,27 +29823,27 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__2; +x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__2; x_2 = l_Lean_Elab_Term_withoutTacticIncrementality___at_Lean_Elab_Tactic_ElimApp_evalAlts_applyPreTac___spec__1___closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__3; +x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__3; x_2 = l_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___lambda__3___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__5() { _start: { lean_object* x_1; @@ -29701,17 +29851,17 @@ x_1 = lean_mk_string_unchecked("initFn", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__6() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__4; -x_2 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__5; +x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__4; +x_2 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__5; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__7() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__7() { _start: { lean_object* x_1; @@ -29719,47 +29869,47 @@ x_1 = lean_mk_string_unchecked("_@", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__8() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__6; -x_2 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__7; +x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__6; +x_2 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__7; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__9() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__8; +x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__8; x_2 = l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getAltName___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__10() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__9; +x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__9; x_2 = l_Lean_Elab_Term_withoutTacticIncrementality___at_Lean_Elab_Tactic_ElimApp_evalAlts_applyPreTac___spec__1___closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__11() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__10; +x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__10; x_2 = l_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___lambda__3___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__12() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__12() { _start: { lean_object* x_1; @@ -29767,17 +29917,17 @@ x_1 = lean_mk_string_unchecked("Induction", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__13() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__11; -x_2 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__12; +x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__11; +x_2 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__12; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__14() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__14() { _start: { lean_object* x_1; @@ -29785,33 +29935,33 @@ x_1 = lean_mk_string_unchecked("_hyg", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__15() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__13; -x_2 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__14; +x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__13; +x_2 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__14; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__16() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__16() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__15; -x_2 = lean_unsigned_to_nat(11137u); +x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__15; +x_2 = lean_unsigned_to_nat(11161u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161_(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; -x_2 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__1; +x_2 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__1; x_3 = 0; -x_4 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__16; +x_4 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__16; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); if (lean_obj_tag(x_5) == 0) { @@ -30086,19 +30236,19 @@ l_Lean_Elab_Tactic_getInductiveValFromMajor___lambda__1___closed__2 = _init_l_Le lean_mark_persistent(l_Lean_Elab_Tactic_getInductiveValFromMajor___lambda__1___closed__2); l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_elabTermForElim___closed__1 = _init_l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_elabTermForElim___closed__1(); lean_mark_persistent(l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_elabTermForElim___closed__1); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__1 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__1); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__2 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__2); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__3 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__3); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__4 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__4); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__5 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__5); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__6 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__6); -if (builtin) {res = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079_(lean_io_mk_world()); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__1 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__1); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__2 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__2); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__3 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__3); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__4 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__4); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__5 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__5); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__6 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__6); +if (builtin) {res = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_Elab_Tactic_tactic_customEliminators = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Elab_Tactic_tactic_customEliminators); @@ -30227,39 +30377,39 @@ lean_dec_ref(res); }if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_evalCases__2(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__1 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__1); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__2 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__2); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__3 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__3); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__4 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__4); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__5 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__5); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__6 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__6); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__7 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__7); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__8 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__8(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__8); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__9 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__9(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__9); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__10 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__10(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__10); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__11 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__11(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__11); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__12 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__12(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__12); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__13 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__13(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__13); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__14 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__14(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__14); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__15 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__15(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__15); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__16 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__16(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__16); -if (builtin) {res = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137_(lean_io_mk_world()); +}l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__1 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__1); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__2 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__2); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__3 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__3); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__4 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__4); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__5 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__5); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__6 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__6); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__7 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__7); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__8 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__8(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__8); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__9 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__9(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__9); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__10 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__10(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__10); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__11 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__11(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__11); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__12 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__12(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__12); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__13 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__13(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__13); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__14 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__14(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__14); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__15 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__15(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__15); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__16 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__16(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__16); +if (builtin) {res = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }return lean_io_result_mk_ok(lean_box(0)); diff --git a/stage0/stdlib/Lean/Elab/Tactic/SolveByElim.c b/stage0/stdlib/Lean/Elab/Tactic/SolveByElim.c index e79d6443eb49..2ea2ccd5c9b9 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/SolveByElim.c +++ b/stage0/stdlib/Lean/Elab/Tactic/SolveByElim.c @@ -173,6 +173,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_SolveByElim_evalApplyRu static lean_object* l_Lean_Elab_Tactic_SolveByElim_elabConfig___closed__1; lean_object* l_Sum_getLeft_x3f___rarg(lean_object*); lean_object* l_Lean_throwError___at_Lean_Meta_mkSimpCongrTheorem___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Sum_Basic_0__Sum_beqSum____x40_Init_Data_Sum_Basic___hyg_243____at_Lean_Elab_Tactic_SolveByElim_parseArgs___spec__5___boxed(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_SolveByElim_evalApplyAssumption_declRange__1___closed__1; static lean_object* l_Lean_Elab_Tactic_SolveByElim_elabConfig___closed__8; static lean_object* l___regBuiltin_Lean_Elab_Tactic_SolveByElim_evalApplyRules_declRange__1___closed__4; @@ -212,7 +213,6 @@ static lean_object* l_Lean_Elab_Tactic_SolveByElim_evalApplyRules___closed__2; LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapMAux___at_Lean_Elab_Tactic_SolveByElim_elabConfig___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_SolveByElim_elabConfig___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT uint8_t l___private_Init_Data_Sum_0__Sum_beqSum____x40_Init_Data_Sum___hyg_242____at_Lean_Elab_Tactic_SolveByElim_parseArgs___spec__5(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_SolveByElim_evalSolveByElim___lambda__1(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static size_t l_Lean_Elab_Tactic_SolveByElim_parseArgs___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Tactic_SolveByElim_evalApplyAssumption_declRange__1___closed__2; @@ -226,7 +226,6 @@ size_t lean_usize_add(size_t, size_t); static lean_object* l_Lean_Elab_withSaveInfoContext___at_Lean_Elab_Tactic_SolveByElim_elabConfig___spec__1___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Tactic_SolveByElim_evalApplyAssumption_declRange__1___closed__6; static lean_object* l_Lean_Elab_Tactic_SolveByElim_parseUsing___closed__1; -LEAN_EXPORT lean_object* l___private_Init_Data_Sum_0__Sum_beqSum____x40_Init_Data_Sum___hyg_242____at_Lean_Elab_Tactic_SolveByElim_parseArgs___spec__5___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_withoutModifyingStateWithInfoAndMessages___at_Lean_Elab_Tactic_SolveByElim_elabConfig___spec__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_SolveByElim_processSyntax(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_SolveByElim_elabApplyRulesConfig(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -242,6 +241,7 @@ static lean_object* l_Lean_Elab_Tactic_SolveByElim_elabConfig___closed__13; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_SolveByElim_processSyntax___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_evalExpr_x27___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_SolveByElim_evalUnsafe____x40_Lean_Elab_Tactic_SolveByElim___hyg_8____closed__4; +LEAN_EXPORT uint8_t l___private_Init_Data_Sum_Basic_0__Sum_beqSum____x40_Init_Data_Sum_Basic___hyg_243____at_Lean_Elab_Tactic_SolveByElim_parseArgs___spec__5(lean_object*, lean_object*); extern lean_object* l_Lean_Elab_unsupportedSyntaxExceptionId; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_SolveByElim_evalUnsafe____x40_Lean_Elab_Tactic_SolveByElim___hyg_8____boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); @@ -3612,7 +3612,7 @@ goto _start; } } } -LEAN_EXPORT uint8_t l___private_Init_Data_Sum_0__Sum_beqSum____x40_Init_Data_Sum___hyg_242____at_Lean_Elab_Tactic_SolveByElim_parseArgs___spec__5(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l___private_Init_Data_Sum_Basic_0__Sum_beqSum____x40_Init_Data_Sum_Basic___hyg_243____at_Lean_Elab_Tactic_SolveByElim_parseArgs___spec__5(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -3700,7 +3700,7 @@ lean_dec(x_1); x_7 = lean_ctor_get(x_2, 0); lean_inc(x_7); lean_dec(x_2); -x_8 = l___private_Init_Data_Sum_0__Sum_beqSum____x40_Init_Data_Sum___hyg_242____at_Lean_Elab_Tactic_SolveByElim_parseArgs___spec__5(x_6, x_7); +x_8 = l___private_Init_Data_Sum_Basic_0__Sum_beqSum____x40_Init_Data_Sum_Basic___hyg_243____at_Lean_Elab_Tactic_SolveByElim_parseArgs___spec__5(x_6, x_7); return x_8; } } @@ -3988,11 +3988,11 @@ x_6 = l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_SolveByElim_parseArgs___spec_ return x_6; } } -LEAN_EXPORT lean_object* l___private_Init_Data_Sum_0__Sum_beqSum____x40_Init_Data_Sum___hyg_242____at_Lean_Elab_Tactic_SolveByElim_parseArgs___spec__5___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Init_Data_Sum_Basic_0__Sum_beqSum____x40_Init_Data_Sum_Basic___hyg_243____at_Lean_Elab_Tactic_SolveByElim_parseArgs___spec__5___boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l___private_Init_Data_Sum_0__Sum_beqSum____x40_Init_Data_Sum___hyg_242____at_Lean_Elab_Tactic_SolveByElim_parseArgs___spec__5(x_1, x_2); +x_3 = l___private_Init_Data_Sum_Basic_0__Sum_beqSum____x40_Init_Data_Sum_Basic___hyg_243____at_Lean_Elab_Tactic_SolveByElim_parseArgs___spec__5(x_1, x_2); x_4 = lean_box(x_3); return x_4; } diff --git a/stage0/stdlib/Lean/Elab/Tactic/Unfold.c b/stage0/stdlib/Lean/Elab/Tactic/Unfold.c index fea9a8afe4ca..bd5fc6fd0d09 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/Unfold.c +++ b/stage0/stdlib/Lean/Elab/Tactic/Unfold.c @@ -19,29 +19,33 @@ lean_object* l_Lean_Meta_throwTacticEx___rarg(lean_object*, lean_object*, lean_o lean_object* l_Lean_addBuiltinDocString(lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalUnfold_declRange__1___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_zetaDeltaLocalDecl___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_evalUnfold_go___lambda__4___closed__8; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_unfoldLocalDecl(lean_object*, 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_evalUnfold__1___closed__1; lean_object* l_Lean_Elab_Tactic_expandOptLocation(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_unfoldLocalDecl___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Elab_Tactic_tacticElabAttribute; +lean_object* l_Lean_FVarId_isLetVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getArgs(lean_object*); lean_object* l_Lean_replaceRef(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalUnfold__1___closed__9; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalUnfold__1___closed__2; 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_evalUnfold_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_EXPORT lean_object* l_Lean_Elab_Tactic_evalUnfold_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_EXPORT lean_object* l_Lean_Elab_Tactic_unfoldTarget___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_evalUnfold_go___lambda__1___closed__3; lean_object* l_Lean_addBuiltinDeclarationRanges(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalUnfold(lean_object*, lean_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_evalUnfold_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*); +static lean_object* l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__5; lean_object* l_Lean_Meta_zetaDeltaTarget(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_zetaDeltaLocalDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_stringToMessageData(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalUnfold_docString__1___closed__1; -static lean_object* l_Lean_Elab_Tactic_evalUnfold_go___lambda__3___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalUnfold__1___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalUnfold_declRange__1___closed__7; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalUnfold_go___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_withLocation(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalUnfold_docString__1(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalUnfold__1___closed__3; @@ -54,10 +58,11 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalUnfo lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalUnfold__1___closed__5; -static lean_object* l_Lean_Elab_Tactic_evalUnfold_go___lambda__3___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalUnfold___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofExpr(lean_object*); static lean_object* l_Lean_Elab_Tactic_evalUnfold_go___lambda__1___closed__6; +static lean_object* l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__3; +static lean_object* l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalUnfold_declRange__1___closed__6; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalUnfold__1___closed__7; static lean_object* l_Lean_Elab_Tactic_evalUnfold_go___lambda__1___closed__5; @@ -65,18 +70,21 @@ static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalUnfold__1___closed__8; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalUnfold__1(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_Elab_Tactic_zetaDeltaTarget(lean_object*, 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_evalUnfold_go___lambda__4___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalUnfold_declRange__1___closed__1; -static lean_object* l_Lean_Elab_Tactic_evalUnfold_go___lambda__3___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalUnfold_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*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalUnfold_declRange__1___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalUnfold_declRange__1___closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalUnfold_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*); +static lean_object* l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__6; +static lean_object* l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__7; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalUnfold_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*); size_t lean_usize_add(size_t, size_t); lean_object* lean_array_uget(lean_object*, size_t); +lean_object* l_Lean_Expr_fvar___override(lean_object*); static lean_object* l_Lean_Elab_Tactic_evalUnfold_go___lambda__1___closed__1; size_t lean_array_size(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_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_evalUnfold_go___lambda__3___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_zetaDeltaTarget___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_evalUnfold___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_evalUnfold_go___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -89,6 +97,7 @@ lean_object* l_Lean_Meta_unfoldTarget(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___regBuiltin_Lean_Elab_Tactic_evalUnfold__1___closed__6; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalUnfold_declRange__1(lean_object*); +static lean_object* l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_unfoldLocalDecl(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, 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: { @@ -583,7 +592,22 @@ x_19 = l_Lean_Meta_throwTacticEx___rarg(x_18, x_2, x_17, x_7, x_8, x_9, x_10, x_ return x_19; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalUnfold_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_EXPORT lean_object* l_Lean_Elab_Tactic_evalUnfold_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) { +_start: +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +lean_inc(x_1); +x_14 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_zetaDeltaLocalDecl___boxed), 11, 1); +lean_closure_set(x_14, 0, x_1); +x_15 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_zetaDeltaTarget___boxed), 10, 1); +lean_closure_set(x_15, 0, x_1); +x_16 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalUnfold_go___lambda__1___boxed), 11, 1); +lean_closure_set(x_16, 0, x_2); +x_17 = l_Lean_Elab_Tactic_withLocation(x_3, x_14, x_15, x_16, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +return x_17; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalUnfold_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) { _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; @@ -603,7 +627,7 @@ x_19 = l_Lean_Meta_throwTacticEx___rarg(x_18, x_2, x_17, x_7, x_8, x_9, x_10, x_ return x_19; } } -static lean_object* _init_l_Lean_Elab_Tactic_evalUnfold_go___lambda__3___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__1() { _start: { lean_object* x_1; @@ -611,16 +635,16 @@ x_1 = lean_mk_string_unchecked("expression ", 11, 11); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_evalUnfold_go___lambda__3___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Tactic_evalUnfold_go___lambda__3___closed__1; +x_1 = l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Tactic_evalUnfold_go___lambda__3___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__3() { _start: { lean_object* x_1; @@ -628,20 +652,62 @@ x_1 = lean_mk_string_unchecked(" is not a global or local constant", 34, 34); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_evalUnfold_go___lambda__3___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Tactic_evalUnfold_go___lambda__3___closed__3; +x_1 = l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__3; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalUnfold_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) { +static lean_object* _init_l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("tactic 'unfold' failed, local variable '", 40, 40); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__5; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__7() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("' has no definition", 19, 19); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__8() { _start: { -uint8_t x_12; lean_object* x_13; -x_12 = 0; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__7; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalUnfold_go___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, 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; uint8_t x_15; lean_object* x_16; +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 = 0; lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); @@ -650,163 +716,203 @@ lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -lean_inc(x_1); -x_13 = l_Lean_Elab_Tactic_elabTermForApply(x_1, x_12, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_13) == 0) +x_16 = l_Lean_Elab_Tactic_elabTermForApply(x_1, x_15, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_16) == 0) { -lean_object* x_14; -x_14 = lean_ctor_get(x_13, 0); -lean_inc(x_14); -switch (lean_obj_tag(x_14)) { +lean_object* x_17; +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +switch (lean_obj_tag(x_17)) { case 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_dec(x_1); -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_inc(x_16); -x_17 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_zetaDeltaLocalDecl___boxed), 11, 1); -lean_closure_set(x_17, 0, x_16); -x_18 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_zetaDeltaTarget___boxed), 10, 1); -lean_closure_set(x_18, 0, x_16); -x_19 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalUnfold_go___lambda__1___boxed), 11, 1); -lean_closure_set(x_19, 0, x_14); -x_20 = l_Lean_Elab_Tactic_withLocation(x_2, x_17, x_18, x_19, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_15); -return x_20; -} -case 4: +lean_object* x_18; lean_object* x_19; lean_object* x_20; +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_inc(x_7); +lean_inc(x_19); +x_20 = l_Lean_FVarId_isLetVar(x_19, x_7, x_8, x_9, x_10, x_18); +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_dec(x_1); -x_21 = lean_ctor_get(x_13, 1); +lean_object* x_21; uint8_t x_22; +x_21 = lean_ctor_get(x_20, 0); lean_inc(x_21); -lean_dec(x_13); -x_22 = lean_ctor_get(x_14, 0); -lean_inc(x_22); -lean_dec(x_14); -lean_inc(x_22); -x_23 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_unfoldLocalDecl___boxed), 11, 1); -lean_closure_set(x_23, 0, x_22); -lean_inc(x_22); -x_24 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_unfoldTarget___boxed), 10, 1); -lean_closure_set(x_24, 0, x_22); -x_25 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalUnfold_go___lambda__2___boxed), 11, 1); -lean_closure_set(x_25, 0, x_22); -x_26 = l_Lean_Elab_Tactic_withLocation(x_2, x_23, x_24, x_25, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_21); -return x_26; +x_22 = lean_unbox(x_21); +lean_dec(x_21); +if (x_22 == 0) +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; 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_dec(x_17); +x_23 = lean_ctor_get(x_20, 1); +lean_inc(x_23); +lean_dec(x_20); +x_24 = l_Lean_Expr_fvar___override(x_19); +x_25 = l_Lean_MessageData_ofExpr(x_24); +x_26 = l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__6; +x_27 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_25); +x_28 = l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__8; +x_29 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_29, 0, x_27); +lean_ctor_set(x_29, 1, x_28); +x_30 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(x_29, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_23); +lean_dec(x_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_31 = !lean_is_exclusive(x_30); +if (x_31 == 0) +{ +return x_30; } -default: +else { -lean_object* x_27; lean_object* x_28; -x_27 = lean_ctor_get(x_13, 1); -lean_inc(x_27); -lean_dec(x_13); -x_28 = l_Lean_Elab_Tactic_getMainGoal(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_27); +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_30, 0); +x_33 = lean_ctor_get(x_30, 1); +lean_inc(x_33); +lean_inc(x_32); +lean_dec(x_30); +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_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_20, 1); +lean_inc(x_35); +lean_dec(x_20); +x_36 = lean_box(0); +x_37 = l_Lean_Elab_Tactic_evalUnfold_go___lambda__2(x_19, x_17, x_2, x_36, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_35); +return x_37; +} +} +else +{ +uint8_t x_38; +lean_dec(x_19); +lean_dec(x_17); +lean_dec(x_9); +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); -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; uint8_t x_49; lean_object* x_50; uint8_t x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; -x_29 = lean_ctor_get(x_28, 0); -lean_inc(x_29); -x_30 = lean_ctor_get(x_28, 1); -lean_inc(x_30); -lean_dec(x_28); -x_31 = l_Lean_MessageData_ofExpr(x_14); -x_32 = l_Lean_Elab_Tactic_evalUnfold_go___lambda__3___closed__2; -x_33 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_33, 0, x_32); -lean_ctor_set(x_33, 1, x_31); -x_34 = l_Lean_Elab_Tactic_evalUnfold_go___lambda__3___closed__4; -x_35 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_35, 0, x_33); -lean_ctor_set(x_35, 1, x_34); -x_36 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_36, 0, x_35); -x_37 = lean_ctor_get(x_9, 5); -lean_inc(x_37); -x_38 = l_Lean_replaceRef(x_1, x_37); -lean_dec(x_37); -lean_dec(x_1); -x_39 = lean_ctor_get(x_9, 0); -lean_inc(x_39); -x_40 = lean_ctor_get(x_9, 1); +x_38 = !lean_is_exclusive(x_20); +if (x_38 == 0) +{ +return x_20; +} +else +{ +lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = lean_ctor_get(x_20, 0); +x_40 = lean_ctor_get(x_20, 1); lean_inc(x_40); -x_41 = lean_ctor_get(x_9, 2); -lean_inc(x_41); -x_42 = lean_ctor_get(x_9, 3); +lean_inc(x_39); +lean_dec(x_20); +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; +} +} +} +case 4: +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_42 = lean_ctor_get(x_16, 1); lean_inc(x_42); -x_43 = lean_ctor_get(x_9, 4); +lean_dec(x_16); +x_43 = lean_ctor_get(x_17, 0); +lean_inc(x_43); +lean_dec(x_17); lean_inc(x_43); -x_44 = lean_ctor_get(x_9, 6); -lean_inc(x_44); -x_45 = lean_ctor_get(x_9, 7); -lean_inc(x_45); -x_46 = lean_ctor_get(x_9, 8); -lean_inc(x_46); -x_47 = lean_ctor_get(x_9, 9); -lean_inc(x_47); -x_48 = lean_ctor_get(x_9, 10); +x_44 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_unfoldLocalDecl___boxed), 11, 1); +lean_closure_set(x_44, 0, x_43); +lean_inc(x_43); +x_45 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_unfoldTarget___boxed), 10, 1); +lean_closure_set(x_45, 0, x_43); +x_46 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalUnfold_go___lambda__3___boxed), 11, 1); +lean_closure_set(x_46, 0, x_43); +x_47 = l_Lean_Elab_Tactic_withLocation(x_2, x_44, x_45, x_46, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_42); +return x_47; +} +default: +{ +lean_object* x_48; lean_object* x_49; +x_48 = lean_ctor_get(x_16, 1); lean_inc(x_48); -x_49 = lean_ctor_get_uint8(x_9, sizeof(void*)*12); -x_50 = lean_ctor_get(x_9, 11); +lean_dec(x_16); +x_49 = l_Lean_Elab_Tactic_getMainGoal(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_48); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +if (lean_obj_tag(x_49) == 0) +{ +lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_50 = lean_ctor_get(x_49, 0); lean_inc(x_50); -x_51 = lean_ctor_get_uint8(x_9, sizeof(void*)*12 + 1); -lean_dec(x_9); -x_52 = lean_alloc_ctor(0, 12, 2); -lean_ctor_set(x_52, 0, x_39); -lean_ctor_set(x_52, 1, x_40); -lean_ctor_set(x_52, 2, x_41); -lean_ctor_set(x_52, 3, x_42); -lean_ctor_set(x_52, 4, x_43); -lean_ctor_set(x_52, 5, x_38); -lean_ctor_set(x_52, 6, x_44); -lean_ctor_set(x_52, 7, x_45); -lean_ctor_set(x_52, 8, x_46); -lean_ctor_set(x_52, 9, x_47); -lean_ctor_set(x_52, 10, x_48); -lean_ctor_set(x_52, 11, x_50); -lean_ctor_set_uint8(x_52, sizeof(void*)*12, x_49); -lean_ctor_set_uint8(x_52, sizeof(void*)*12 + 1, x_51); -x_53 = l_Lean_Elab_Tactic_evalUnfold_go___lambda__1___closed__2; -x_54 = l_Lean_Meta_throwTacticEx___rarg(x_53, x_29, x_36, x_7, x_8, x_52, x_10, x_30); +x_51 = lean_ctor_get(x_49, 1); +lean_inc(x_51); +lean_dec(x_49); +x_52 = l_Lean_MessageData_ofExpr(x_17); +x_53 = l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__2; +x_54 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_54, 0, x_53); +lean_ctor_set(x_54, 1, x_52); +x_55 = l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__4; +x_56 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_56, 0, x_54); +lean_ctor_set(x_56, 1, x_55); +x_57 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_57, 0, x_56); +x_58 = l_Lean_Elab_Tactic_evalUnfold_go___lambda__1___closed__2; +x_59 = l_Lean_Meta_throwTacticEx___rarg(x_58, x_50, x_57, x_7, x_8, x_9, x_10, x_51); lean_dec(x_10); -lean_dec(x_52); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -return x_54; +return x_59; } else { -uint8_t x_55; -lean_dec(x_14); -lean_dec(x_10); +uint8_t x_60; +lean_dec(x_17); lean_dec(x_9); +lean_dec(x_10); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_1); -x_55 = !lean_is_exclusive(x_28); -if (x_55 == 0) +x_60 = !lean_is_exclusive(x_49); +if (x_60 == 0) { -return x_28; +return x_49; } else { -lean_object* x_56; lean_object* x_57; lean_object* x_58; -x_56 = lean_ctor_get(x_28, 0); -x_57 = lean_ctor_get(x_28, 1); -lean_inc(x_57); -lean_inc(x_56); -lean_dec(x_28); -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_61; lean_object* x_62; lean_object* x_63; +x_61 = lean_ctor_get(x_49, 0); +x_62 = lean_ctor_get(x_49, 1); +lean_inc(x_62); +lean_inc(x_61); +lean_dec(x_49); +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; } } } @@ -814,33 +920,330 @@ return x_58; } else { -uint8_t x_59; +uint8_t x_64; +lean_dec(x_9); 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); +x_64 = !lean_is_exclusive(x_16); +if (x_64 == 0) +{ +return x_16; +} +else +{ +lean_object* x_65; lean_object* x_66; lean_object* x_67; +x_65 = lean_ctor_get(x_16, 0); +x_66 = lean_ctor_get(x_16, 1); +lean_inc(x_66); +lean_inc(x_65); +lean_dec(x_16); +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_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; uint8_t x_79; lean_object* x_80; uint8_t x_81; lean_object* x_82; lean_object* x_83; uint8_t x_84; lean_object* x_85; +x_68 = lean_ctor_get(x_9, 0); +x_69 = lean_ctor_get(x_9, 1); +x_70 = lean_ctor_get(x_9, 2); +x_71 = lean_ctor_get(x_9, 3); +x_72 = lean_ctor_get(x_9, 4); +x_73 = lean_ctor_get(x_9, 5); +x_74 = lean_ctor_get(x_9, 6); +x_75 = lean_ctor_get(x_9, 7); +x_76 = lean_ctor_get(x_9, 8); +x_77 = lean_ctor_get(x_9, 9); +x_78 = lean_ctor_get(x_9, 10); +x_79 = lean_ctor_get_uint8(x_9, sizeof(void*)*12); +x_80 = lean_ctor_get(x_9, 11); +x_81 = lean_ctor_get_uint8(x_9, sizeof(void*)*12 + 1); +lean_inc(x_80); +lean_inc(x_78); +lean_inc(x_77); +lean_inc(x_76); +lean_inc(x_75); +lean_inc(x_74); +lean_inc(x_73); +lean_inc(x_72); +lean_inc(x_71); +lean_inc(x_70); +lean_inc(x_69); +lean_inc(x_68); lean_dec(x_9); +x_82 = l_Lean_replaceRef(x_1, x_73); +lean_dec(x_73); +x_83 = lean_alloc_ctor(0, 12, 2); +lean_ctor_set(x_83, 0, x_68); +lean_ctor_set(x_83, 1, x_69); +lean_ctor_set(x_83, 2, x_70); +lean_ctor_set(x_83, 3, x_71); +lean_ctor_set(x_83, 4, x_72); +lean_ctor_set(x_83, 5, x_82); +lean_ctor_set(x_83, 6, x_74); +lean_ctor_set(x_83, 7, x_75); +lean_ctor_set(x_83, 8, x_76); +lean_ctor_set(x_83, 9, x_77); +lean_ctor_set(x_83, 10, x_78); +lean_ctor_set(x_83, 11, x_80); +lean_ctor_set_uint8(x_83, sizeof(void*)*12, x_79); +lean_ctor_set_uint8(x_83, sizeof(void*)*12 + 1, x_81); +x_84 = 0; +lean_inc(x_10); +lean_inc(x_83); +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_85 = l_Lean_Elab_Tactic_elabTermForApply(x_1, x_84, x_3, x_4, x_5, x_6, x_7, x_8, x_83, x_10, x_11); +if (lean_obj_tag(x_85) == 0) +{ +lean_object* x_86; +x_86 = lean_ctor_get(x_85, 0); +lean_inc(x_86); +switch (lean_obj_tag(x_86)) { +case 1: +{ +lean_object* x_87; lean_object* x_88; lean_object* x_89; +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_inc(x_7); +lean_inc(x_88); +x_89 = l_Lean_FVarId_isLetVar(x_88, x_7, x_8, x_83, x_10, x_87); +if (lean_obj_tag(x_89) == 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_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_dec(x_86); +x_92 = lean_ctor_get(x_89, 1); +lean_inc(x_92); +lean_dec(x_89); +x_93 = l_Lean_Expr_fvar___override(x_88); +x_94 = l_Lean_MessageData_ofExpr(x_93); +x_95 = l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__6; +x_96 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_96, 0, x_95); +lean_ctor_set(x_96, 1, x_94); +x_97 = l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__8; +x_98 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_98, 0, x_96); +lean_ctor_set(x_98, 1, x_97); +x_99 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(x_98, x_3, x_4, x_5, x_6, x_7, x_8, x_83, x_10, x_92); +lean_dec(x_10); +lean_dec(x_83); lean_dec(x_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_59 = !lean_is_exclusive(x_13); -if (x_59 == 0) +x_100 = lean_ctor_get(x_99, 0); +lean_inc(x_100); +x_101 = lean_ctor_get(x_99, 1); +lean_inc(x_101); +if (lean_is_exclusive(x_99)) { + lean_ctor_release(x_99, 0); + lean_ctor_release(x_99, 1); + x_102 = x_99; +} else { + lean_dec_ref(x_99); + x_102 = lean_box(0); +} +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 { -return x_13; +lean_object* x_104; lean_object* x_105; lean_object* x_106; +x_104 = lean_ctor_get(x_89, 1); +lean_inc(x_104); +lean_dec(x_89); +x_105 = lean_box(0); +x_106 = l_Lean_Elab_Tactic_evalUnfold_go___lambda__2(x_88, x_86, x_2, x_105, x_3, x_4, x_5, x_6, x_7, x_8, x_83, x_10, x_104); +return x_106; +} } else { -lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_60 = lean_ctor_get(x_13, 0); -x_61 = lean_ctor_get(x_13, 1); -lean_inc(x_61); -lean_inc(x_60); -lean_dec(x_13); -x_62 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_62, 0, x_60); -lean_ctor_set(x_62, 1, x_61); -return x_62; +lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; +lean_dec(x_88); +lean_dec(x_86); +lean_dec(x_83); +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); +x_107 = lean_ctor_get(x_89, 0); +lean_inc(x_107); +x_108 = lean_ctor_get(x_89, 1); +lean_inc(x_108); +if (lean_is_exclusive(x_89)) { + lean_ctor_release(x_89, 0); + lean_ctor_release(x_89, 1); + x_109 = x_89; +} else { + lean_dec_ref(x_89); + x_109 = lean_box(0); +} +if (lean_is_scalar(x_109)) { + x_110 = lean_alloc_ctor(1, 2, 0); +} else { + x_110 = x_109; +} +lean_ctor_set(x_110, 0, x_107); +lean_ctor_set(x_110, 1, x_108); +return x_110; +} +} +case 4: +{ +lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; +x_111 = lean_ctor_get(x_85, 1); +lean_inc(x_111); +lean_dec(x_85); +x_112 = lean_ctor_get(x_86, 0); +lean_inc(x_112); +lean_dec(x_86); +lean_inc(x_112); +x_113 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_unfoldLocalDecl___boxed), 11, 1); +lean_closure_set(x_113, 0, x_112); +lean_inc(x_112); +x_114 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_unfoldTarget___boxed), 10, 1); +lean_closure_set(x_114, 0, x_112); +x_115 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalUnfold_go___lambda__3___boxed), 11, 1); +lean_closure_set(x_115, 0, x_112); +x_116 = l_Lean_Elab_Tactic_withLocation(x_2, x_113, x_114, x_115, x_3, x_4, x_5, x_6, x_7, x_8, x_83, x_10, x_111); +return x_116; +} +default: +{ +lean_object* x_117; lean_object* x_118; +x_117 = lean_ctor_get(x_85, 1); +lean_inc(x_117); +lean_dec(x_85); +x_118 = l_Lean_Elab_Tactic_getMainGoal(x_3, x_4, x_5, x_6, x_7, x_8, x_83, x_10, x_117); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +if (lean_obj_tag(x_118) == 0) +{ +lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; +x_119 = lean_ctor_get(x_118, 0); +lean_inc(x_119); +x_120 = lean_ctor_get(x_118, 1); +lean_inc(x_120); +lean_dec(x_118); +x_121 = l_Lean_MessageData_ofExpr(x_86); +x_122 = l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__2; +x_123 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_123, 0, x_122); +lean_ctor_set(x_123, 1, x_121); +x_124 = l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__4; +x_125 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_125, 0, x_123); +lean_ctor_set(x_125, 1, x_124); +x_126 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_126, 0, x_125); +x_127 = l_Lean_Elab_Tactic_evalUnfold_go___lambda__1___closed__2; +x_128 = l_Lean_Meta_throwTacticEx___rarg(x_127, x_119, x_126, x_7, x_8, x_83, x_10, x_120); +lean_dec(x_10); +lean_dec(x_83); +lean_dec(x_8); +lean_dec(x_7); +return x_128; +} +else +{ +lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; +lean_dec(x_86); +lean_dec(x_83); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_7); +x_129 = lean_ctor_get(x_118, 0); +lean_inc(x_129); +x_130 = lean_ctor_get(x_118, 1); +lean_inc(x_130); +if (lean_is_exclusive(x_118)) { + lean_ctor_release(x_118, 0); + lean_ctor_release(x_118, 1); + x_131 = x_118; +} else { + lean_dec_ref(x_118); + x_131 = lean_box(0); +} +if (lean_is_scalar(x_131)) { + x_132 = lean_alloc_ctor(1, 2, 0); +} else { + x_132 = x_131; +} +lean_ctor_set(x_132, 0, x_129); +lean_ctor_set(x_132, 1, x_130); +return x_132; +} +} +} +} +else +{ +lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; +lean_dec(x_83); +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); +x_133 = lean_ctor_get(x_85, 0); +lean_inc(x_133); +x_134 = lean_ctor_get(x_85, 1); +lean_inc(x_134); +if (lean_is_exclusive(x_85)) { + lean_ctor_release(x_85, 0); + lean_ctor_release(x_85, 1); + x_135 = x_85; +} else { + lean_dec_ref(x_85); + x_135 = lean_box(0); +} +if (lean_is_scalar(x_135)) { + x_136 = lean_alloc_ctor(1, 2, 0); +} else { + x_136 = x_135; +} +lean_ctor_set(x_136, 0, x_133); +lean_ctor_set(x_136, 1, x_134); +return x_136; } } } @@ -849,7 +1252,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalUnfold_go(lean_object* x_1, lean _start: { lean_object* x_12; lean_object* x_13; -x_12 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalUnfold_go___lambda__3___boxed), 11, 2); +x_12 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___boxed), 11, 2); lean_closure_set(x_12, 0, x_1); lean_closure_set(x_12, 1, x_2); x_13 = l_Lean_Elab_Tactic_withMainContext___rarg(x_12, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); @@ -872,11 +1275,21 @@ lean_dec(x_3); return x_12; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalUnfold_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_EXPORT lean_object* l_Lean_Elab_Tactic_evalUnfold_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) { +_start: +{ +lean_object* x_14; +x_14 = l_Lean_Elab_Tactic_evalUnfold_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); +lean_dec(x_4); +lean_dec(x_3); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalUnfold_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) { _start: { lean_object* x_12; -x_12 = l_Lean_Elab_Tactic_evalUnfold_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 = l_Lean_Elab_Tactic_evalUnfold_go___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -888,11 +1301,11 @@ lean_dec(x_3); return x_12; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalUnfold_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_EXPORT lean_object* l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { lean_object* x_12; -x_12 = l_Lean_Elab_Tactic_evalUnfold_go___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_12 = l_Lean_Elab_Tactic_evalUnfold_go___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_2); return x_12; } @@ -1310,14 +1723,22 @@ l_Lean_Elab_Tactic_evalUnfold_go___lambda__1___closed__5 = _init_l_Lean_Elab_Tac lean_mark_persistent(l_Lean_Elab_Tactic_evalUnfold_go___lambda__1___closed__5); l_Lean_Elab_Tactic_evalUnfold_go___lambda__1___closed__6 = _init_l_Lean_Elab_Tactic_evalUnfold_go___lambda__1___closed__6(); lean_mark_persistent(l_Lean_Elab_Tactic_evalUnfold_go___lambda__1___closed__6); -l_Lean_Elab_Tactic_evalUnfold_go___lambda__3___closed__1 = _init_l_Lean_Elab_Tactic_evalUnfold_go___lambda__3___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_evalUnfold_go___lambda__3___closed__1); -l_Lean_Elab_Tactic_evalUnfold_go___lambda__3___closed__2 = _init_l_Lean_Elab_Tactic_evalUnfold_go___lambda__3___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_evalUnfold_go___lambda__3___closed__2); -l_Lean_Elab_Tactic_evalUnfold_go___lambda__3___closed__3 = _init_l_Lean_Elab_Tactic_evalUnfold_go___lambda__3___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_evalUnfold_go___lambda__3___closed__3); -l_Lean_Elab_Tactic_evalUnfold_go___lambda__3___closed__4 = _init_l_Lean_Elab_Tactic_evalUnfold_go___lambda__3___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_evalUnfold_go___lambda__3___closed__4); +l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__1 = _init_l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__1); +l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__2 = _init_l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__2); +l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__3 = _init_l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__3); +l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__4 = _init_l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__4); +l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__5 = _init_l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__5); +l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__6 = _init_l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__6); +l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__7 = _init_l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__7); +l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__8 = _init_l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__8(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalUnfold_go___lambda__4___closed__8); l___regBuiltin_Lean_Elab_Tactic_evalUnfold__1___closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_evalUnfold__1___closed__1(); lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_evalUnfold__1___closed__1); l___regBuiltin_Lean_Elab_Tactic_evalUnfold__1___closed__2 = _init_l___regBuiltin_Lean_Elab_Tactic_evalUnfold__1___closed__2(); diff --git a/stage0/stdlib/Lean/Elab/Term.c b/stage0/stdlib/Lean/Elab/Term.c index af6f01980ae7..b8427267ed07 100644 --- a/stage0/stdlib/Lean/Elab/Term.c +++ b/stage0/stdlib/Lean/Elab/Term.c @@ -22,6 +22,7 @@ static lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Term_0__Lean LEAN_EXPORT lean_object* l_Lean_MVarId_isAssigned___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); static lean_object* l_Lean_logAt___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__2___closed__1; +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Term_exposeLevelMVars___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_hasNoImplicitLambdaAnnotation___closed__1; lean_object* l_Lean_Meta_mkSorry(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -46,7 +47,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_setLevelNames___boxed(lean_object*, le LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutErrToSorryImp(lean_object*); static lean_object* l_Lean_Elab_Term_mkExplicitBinder___closed__11; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutTacticIncrementality___rarg___lambda__2(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274_(lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__3(lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Core_transform___at_Lean_Elab_Term_exposeLevelMVars___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_instInhabitedTermElabM___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -54,7 +54,6 @@ lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at___private_Lean_Metava static lean_object* l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Term_expandDeclId___spec__10___closed__1; static lean_object* l_Lean_Elab_Term_getInfoTreeWithContext_x3f___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_resolveLocalName___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__7; LEAN_EXPORT lean_object* l_Lean_Elab_logException___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withLocalContextImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_throwMVarError___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -65,7 +64,6 @@ static lean_object* l_Lean_Elab_Term_getFVarLocalDecl_x21___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabUsingElabFnsAux___lambda__1(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_synthesizeInstMVarCore___lambda__3___closed__1; static lean_object* l_Lean_Elab_Term_mkAuxName___closed__1; -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__1; extern lean_object* l_Lean_instMonadExceptOfExceptionCoreM; LEAN_EXPORT lean_object* l_Lean_Elab_Term_getInfoTreeWithContext_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_resolveId_x3f(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -97,7 +95,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_TacticParsedSnapshot_data(lean_objec LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerMVarErrorCustomInfo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_MVarId_assign___at_Lean_Elab_Term_exprToSyntax___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_withDeclName___spec__8(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__2; static lean_object* l_Lean_Linter_checkDeprecated___at_Lean_Elab_Term_mkConst___spec__3___closed__7; static lean_object* l_Lean_Elab_Term_withExpectedType___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_exposeLevelMVars___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -117,6 +114,8 @@ LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_v LEAN_EXPORT lean_object* l_Lean_Elab_Term_instAddErrorMessageContextTermElabM(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__10(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_commitIfNoErrors_x3f(lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__11; +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__2; LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_withoutModifyingStateWithInfoAndMessagesImpl___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Core_transform_visit___at_Lean_Elab_Term_exposeLevelMVars___spec__2___boxed__const__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withSavedContext(lean_object*); @@ -133,12 +132,12 @@ static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabUsingElabFn LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_Term_isLetRecAuxMVar___spec__3(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_LevelMVarErrorInfo_logError___lambda__1___closed__4; lean_object* l_Lean_Elab_Level_elabLevel(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__9; LEAN_EXPORT lean_object* l_Lean_Elab_Term_instMonadMacroAdapterTermElabM; LEAN_EXPORT lean_object* l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at_Lean_Elab_Term_withDeclName___spec__2___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_getInfoTreeWithContext_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Core_transform___at_Lean_Elab_Term_exposeLevelMVars___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkTacticMVar___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_Term_isLetRecAuxMVar___lambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_find___at_Lean_Elab_Term_resolveLocalName___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_mkExplicitBinder___closed__6; @@ -153,14 +152,13 @@ lean_object* l_Lean_profileitIOUnsafe___rarg(lean_object*, lean_object*, lean_ob LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_instInhabitedSyntheticMVarDecl; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutTacticIncrementality___rarg(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_mkAuxName___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_RBNode_findCore___at___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_elimApp___spec__4(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instInhabitedTacticParsedSnapshot; LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerSyntheticMVar___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerSyntheticMVarWithCurrRef(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___lambda__4(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withLevelNames(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__34___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_tryPostponeIfHasMVars___closed__4; @@ -170,6 +168,7 @@ static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_expandDeclId___ static lean_object* l_Lean_Elab_Term_synthesizeInstMVarCore___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_beqCacheKey____x40_Lean_Elab_Term___hyg_847____boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutHeedElabAsElim(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__6; uint8_t l_Array_contains___at_Lean_Meta_arrowDomainsN___spec__2(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_instToStringMVarErrorKind___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Term_resolveLocalName_go___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -178,8 +177,8 @@ lean_object* l_Lean_Meta_isProp(lean_object*, lean_object*, lean_object*, lean_o lean_object* l_Lean_ConstantInfo_levelParams(lean_object*); lean_object* l_Lean_indentD(lean_object*); double lean_float_div(double, double); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__7; static lean_object* l_Lean_Elab_Tactic_instBEqCacheKey___closed__1; +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__6; static lean_object* l_Lean_Elab_Term_levelMVarToParam___closed__2; LEAN_EXPORT lean_object* l_Lean_MVarId_withContext___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_synthesizeInstMVarCore___lambda__3___closed__2; @@ -188,8 +187,8 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAu static lean_object* l_Lean_Elab_Tactic_instInhabitedCache___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_useImplicitLambda___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_addDocString___at_Lean_Elab_Term_expandDeclId___spec__9___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint64_t lean_uint64_of_nat(lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3___closed__1; uint64_t lean_uint64_mix_hash(uint64_t, uint64_t); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__41(lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__7(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -218,7 +217,6 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_throwTypeMismatch LEAN_EXPORT lean_object* l_List_filterTR_loop___at_Lean_Elab_Term_resolveId_x3f___spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__4___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutTacticReuse___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__4; static lean_object* l_Lean_Elab_Term_mkCoe___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_instMonadTermElabM___closed__3; @@ -235,8 +233,9 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkCoe___lambda__1(lean_object*, lean_o LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_expandDeclId___spec__4(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MetavarContext_getDelayedMVarAssignmentCore_x3f(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_withRestoreOrSaveFull___rarg___closed__3; -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__3; lean_object* l_Lean_Syntax_getId(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabTermEnsuringType(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at_Lean_Elab_Term_resolveLocalName___spec__5(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); @@ -245,7 +244,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerMVarErrorHoleInfo___boxed(lean LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Term_0__Lean_Elab_Term_withoutModifyingStateWithInfoAndMessagesImpl___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_isLocalIdent_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__41___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__2; lean_object* l_Lean_Expr_sort___override(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_instMonadMacroAdapterTermElabM___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Term_expandDeclId___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -263,25 +261,27 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkConst___lambda__1___boxed(lean_objec LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Term_logUnassignedLevelMVarsUsingErrorInfos___spec__4(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_withDeclName___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_forallBoundedTelescope___at_Lean_Elab_Term_addAutoBoundImplicits_x27___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__4; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___lambda__2___boxed__const__1; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_mkConst___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isNoImplicitLambda___closed__2; lean_object* l_String_removeLeadingSpaces(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_resolveLocalName(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_expandDeclId___spec__4___closed__1; -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__10; lean_object* l_Lean_Core_getMessageLog___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_expandDeclId___closed__1; lean_object* l_Lean_Core_checkSystem(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_Term_resolveId_x3f___spec__3(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_findSomeRevMAux___at_Lean_Elab_Term_resolveLocalName___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_liftExcept___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__8(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20064____closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static double l_Lean_withTraceNode___at_Lean_Elab_Term_mkCoe___spec__1___lambda__4___closed__5; LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__36___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_resolveId_x3f___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_TacticParsedSnapshot_data___boxed(lean_object*); static lean_object* l_Lean_Elab_Term_ensureType___lambda__1___closed__1; +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__5; LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_addTraceNode___at_Lean_Elab_Term_mkCoe___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_mk_array(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_traceAtCmdPos___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -294,6 +294,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_throwAutoBoundImplicitLocal___at_Lean_Elab_ LEAN_EXPORT lean_object* l_Lean_Elab_Term_instToStringMVarErrorKind___boxed(lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Elab_Term_resolveLocalName___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Elab_Term_0__Lean_Elab_Term_isExplicit(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_TermElabM_toIO___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Term_expandDeclId___spec__2___closed__2; @@ -301,7 +302,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_CommandContextInfo_saveNoFileMap___at_Lean_ static lean_object* l_Lean_Elab_getResetInfoTrees___at_Lean_Elab_Term_withDeclName___spec__3___rarg___closed__2; static lean_object* l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__4; static lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Term_expandDeclId___spec__2___lambda__2___closed__1; -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_instMonadTermElabM; lean_object* l_Lean_instMonadQuotationOfMonadFunctorOfMonadLift___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_PersistentArray_anyM___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__5(lean_object*, lean_object*); @@ -315,6 +315,7 @@ lean_object* l_Lean_Expr_mdata___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_hasNoImplicitLambdaAnnotation___boxed(lean_object*); lean_object* l_Lean_Level_isMVar___boxed(lean_object*); static lean_object* l_Lean_Elab_CommandContextInfo_saveNoFileMap___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__3___rarg___closed__1; +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__8; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withNarrowedTacticReuse___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_findSomeRevMAux___at_Lean_Elab_Term_resolveLocalName___spec__4(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_mkAuxName___closed__2; @@ -372,7 +373,7 @@ lean_object* l_Lean_Expr_fvarId_x21(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__38___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Core_transform_visit___at_Lean_Elab_Term_exposeLevelMVars___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_ReaderT_pure___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__12___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__5; +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__15; LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_useImplicitLambda___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_logException___at_Lean_Elab_Term_exceptionToSorry___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_getResetInfoTrees___at_Lean_Elab_Term_withDeclName___spec__3___rarg___closed__1; @@ -405,7 +406,6 @@ static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_dropTermParens_ LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_hashCacheKey____x40_Lean_Elab_Term___hyg_921____boxed(lean_object*); static lean_object* l_Lean_Elab_Term_extraMsgToMsg___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutHeedElabAsElim___rarg(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3___closed__2; static lean_object* l_Lean_Elab_Term_instMonadBacktrackSavedStateTermElabM___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_useImplicitLambda(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Linter_getLinterValue(lean_object*, lean_object*); @@ -426,7 +426,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_throwMVa lean_object* l_Lean_Expr_setPPUniverses(lean_object*, uint8_t); static lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError___closed__3; static lean_object* l_Lean_Elab_Term_withRestoreOrSaveFull___rarg___closed__14; -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__3; lean_object* lean_io_get_num_heartbeats(lean_object*); uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); static lean_object* l_Lean_Linter_checkDeprecated___at_Lean_Elab_Term_mkConst___spec__3___closed__4; @@ -456,7 +455,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutHeedElabAsElim___rarg___lambda_ static lean_object* l_Lean_Elab_Term_instInhabitedMVarErrorKind___closed__7; lean_object* l_Lean_PersistentArray_toList___rarg(lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_Term_getFVarLocalDecl_x21___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__4; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_resolveName_x27___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_List_any___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_synthesizeInstMVarCore___closed__5; @@ -492,7 +490,6 @@ LEAN_EXPORT lean_object* l_Lean_Core_transform_visit_visitPost___at_Lean_Elab_Te static lean_object* l_Lean_Elab_Term_instInhabitedLevelMVarErrorInfo___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__10___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Name_isPrefixOf(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__8; LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__30___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabImplicitLambda_loop___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_instMonadMacroAdapterTermElabM___closed__2; @@ -519,6 +516,7 @@ LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Term_logUnassignedUsin LEAN_EXPORT lean_object* l_Lean_mkAuxName___at_Lean_Elab_Term_mkAuxName___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabImplicitLambdaAux___closed__2; static lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Term_0__Lean_Elab_Term_isLambdaWithImplicit___spec__1___closed__3; +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__3; static lean_object* l_Lean_Elab_Term_tryPostponeIfHasMVars___closed__3; static lean_object* l_Lean_Elab_addBuiltinIncrementalElab___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_tryPostpone___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -532,7 +530,7 @@ lean_object* l_List_mapTR_loop___at_Lean_mkConstWithLevelParams___spec__1(lean_o LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkExplicitBinder(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_instToStringSyntheticMVarKind___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__7; +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__2___closed__2; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__40___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_isLocalIdent_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoTree___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -542,6 +540,7 @@ static lean_object* l_Lean_Elab_Term_synthesizeInstMVarCore___lambda__3___closed LEAN_EXPORT lean_object* l_Lean_Elab_Term_withPushMacroExpansionStack___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Kernel_isDiagnosticsEnabled(lean_object*); static lean_object* l_Lean_Elab_Term_mkTypeMismatchError___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850_(lean_object*); LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_Term_resolveName_x27___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Term_expandDeclId___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabTermEnsuringType___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -550,11 +549,12 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabImplic uint8_t l_Lean_Expr_hasMVar(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instInhabitedCacheKey; uint8_t l_Lean_isReservedName(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_withMacroExpansionInfo___at_Lean_Elab_Term_withMacroExpansion___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__1; static lean_object* l_Lean_Elab_Tactic_instInhabitedTacticFinishedSnapshot___closed__2; static lean_object* l_Lean_Elab_Term_synthesizeInstMVarCore___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Term_TermElabM_run(lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__9; LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isTypeAscription(lean_object*); LEAN_EXPORT uint8_t l_Lean_logAt___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__2___lambda__2(lean_object*); LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -579,7 +579,6 @@ static lean_object* l_Lean_Elab_Term_instInhabitedSyntheticMVarDecl___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutHeedElabAsElimImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_tryPostponeIfHasMVars___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__8; static lean_object* l_Lean_Elab_Term_instMonadMacroAdapterTermElabM___closed__3; lean_object* lean_io_promise_resolve(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabUsingElabFnsAux___lambda__1___closed__1; @@ -627,6 +626,7 @@ static lean_object* l_Lean_Linter_checkDeprecated___at_Lean_Elab_Term_mkConst___ LEAN_EXPORT uint8_t l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___lambda__8(lean_object*); uint8_t l_List_elem___at_Lean_addAliasEntry___spec__16(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_PersistentArray_anyM___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__13(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Term_applyResult___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_withoutHeedElabAsElim___rarg___closed__1; static lean_object* l_Lean_Elab_Term_isLetRecAuxMVar___closed__2; @@ -647,15 +647,14 @@ lean_object* lean_st_ref_take(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_getLetRecsToLift(lean_object*); lean_object* l_Lean_Meta_withRestoreOrSaveFull___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_saveContext(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withReuseContext___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_resolveGlobalName___at_Lean_Elab_Term_resolveLocalName_loop___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Term_expandDeclId___spec__6___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at_Lean_Elab_Term_withDeclName___spec__2___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__4; lean_object* l_liftExcept___at_Lean_Elab_liftMacroM___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_withInfoTreeContext___at_Lean_Elab_Term_withMacroExpansion___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutErrToSorry___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__5; static lean_object* l_Lean_Elab_Term_collectUnassignedMVars_go___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withNarrowedTacticReuse___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_expandMacroImpl_x3f(lean_object*, lean_object*, lean_object*, lean_object*); @@ -663,6 +662,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_TermElabM_toIO___rarg___lambda__1(lean LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkInstMVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_beqCacheKey____x40_Lean_Elab_Term___hyg_847_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__14___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__2; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__31___boxed(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_expr_eqv(lean_object*, lean_object*); lean_object* l_Lean_declareBuiltin(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -671,7 +671,6 @@ lean_object* l_Lean_ResolveName_resolveNamespace(lean_object*, lean_object*, lea lean_object* l_Lean_mkPrivateName(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_exposeLevelMVars___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Term_addDotCompletionInfo___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__4; LEAN_EXPORT lean_object* l_Lean_logWarning___at_Lean_Elab_Term_mkConst___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_tryPostponeIfHasMVars_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Term_0__Lean_Elab_Term_withoutModifyingStateWithInfoAndMessagesImpl___spec__11(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -687,24 +686,27 @@ uint64_t lean_uint64_shift_right(uint64_t, uint64_t); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_instantiateMVars___at___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitMain___spec__7(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withMacroExpansion(lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__1; lean_object* l_Lean_SourceInfo_fromRef(lean_object*, uint8_t); static lean_object* l_Lean_Elab_Term_synthesizeInstMVarCore___lambda__2___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_exposeLevelMVars___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__13; LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__40(lean_object*, lean_object*, size_t, size_t); uint8_t l_Lean_TagAttribute_hasTag(lean_object*, lean_object*, lean_object*); lean_object* l_List_findSome_x3f___rarg(lean_object*, lean_object*); lean_object* l_Lean_Meta_isType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofSyntax(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_resolveName_process(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___closed__3; LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__28___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732_(lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__9(lean_object*, lean_object*, size_t, size_t); lean_object* l_StateRefT_x27_lift___rarg___boxed(lean_object*, lean_object*); lean_object* lean_nat_div(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_getLevelNames(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_logUnassignedLevelMVarsUsingErrorInfos___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedLevelMVarsUsingErrorInfos___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__14; LEAN_EXPORT lean_object* l_Lean_getConstInfo___at_Lean_Elab_Term_mkConst___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__4___boxed(lean_object*, lean_object*, lean_object*); @@ -713,8 +715,8 @@ LEAN_EXPORT uint8_t l_Lean_PersistentArray_anyMAux___at_Lean_Elab_Term_addAutoBo LEAN_EXPORT lean_object* l_Lean_Elab_Term_withNarrowedArgTacticReuse(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instInhabitedCache; LEAN_EXPORT lean_object* l_Lean_Core_transform_visit___at_Lean_Elab_Term_exposeLevelMVars___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__2; lean_object* l_Lean_Option_get___at_Lean_profiler_threshold_getSecs___spec__1(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__9; static lean_object* l_Lean_getConstInfo___at_Lean_Elab_Term_mkConst___spec__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortCommand___at_Lean_Elab_Term_ensureNoUnassignedMVars___spec__1___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutErrToSorryImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -731,6 +733,7 @@ LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Term lean_object* l_Lean_registerTraceClass(lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabUsingElabFnsAux___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instToSnapshotTreeTacticFinishedSnapshot(lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__10; LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_useImplicitLambda___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Term_mkCoe___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_log___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__9(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -741,7 +744,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_TermElabM_toIO(lean_object*); lean_object* l_Lean_Meta_SavedState_restore(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_withSaveInfoContext___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withLocalDeclImp___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__9; LEAN_EXPORT lean_object* l_Lean_Elab_Term_ppGoal(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_tryPostponeIfHasMVars_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__10___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -752,7 +754,6 @@ static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_postponeElabTer static lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withRestoreOrSaveFull___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_mkExplicitBinder___closed__10; -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__9; LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabTerm___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__23(lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Term_expandDeclId___spec__6___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -767,6 +768,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerSyntheticMVarWithCurrRef___box LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__29___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__52(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutMacroStackAtErr___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__12; lean_object* l_Lean_Syntax_getKind(lean_object*); static lean_object* l_Lean_Elab_Term_exposeLevelMVars___lambda__2___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Term_collectUnassignedMVars_go(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -795,7 +797,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_decorateEr LEAN_EXPORT lean_object* l_Lean_Elab_Term_withAuxDecl(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__5___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instToSnapshotTreeTacticParsedSnapshot_go___lambda__1(lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__11; +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_addTermInfo___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_FVarId_getDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -827,7 +829,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_withPushMacroExpansionStack(lean_objec LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Term_mkCoe___spec__1___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_throwMVarError(lean_object*); lean_object* l_Lean_throwError___at_Lean_registerTagAttribute___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__6; uint64_t l___private_Lean_Expr_0__Lean_hashMVarId____x40_Lean_Expr___hyg_1976_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError_appendExtra___boxed(lean_object*, lean_object*); @@ -839,16 +840,16 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerCustomErrorIfMVar___boxed(lean LEAN_EXPORT lean_object* l_Lean_profileitM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__11___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_TermElabM_run_x27___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___boxed__const__1; LEAN_EXPORT lean_object* l_Lean_Elab_addBuiltinIncrementalElab(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_mkFreshBinderName___rarg___closed__1; static lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError___lambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Term_synthesizeInstMVarCore___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_List_isEmpty___rarg(lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__3; +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__4; static lean_object* l_Lean_Elab_Term_instMonadTermElabM___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_traceAtCmdPos(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__6; static uint8_t l_Lean_Elab_Term_collectUnassignedMVars_go___closed__1; static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_mkSyntheticSorryFor___closed__1; static lean_object* l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_throwMVarError___spec__2___rarg___closed__1; @@ -875,13 +876,13 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_termElabAttribute; LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabImplicitLambdaAux___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withMVarContextImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_MessageData_hasTag(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__2; static lean_object* l_Lean_Elab_Term_instToStringSyntheticMVarKind___closed__2; static lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Term_expandDeclId___spec__2___lambda__2___closed__2; static lean_object* l_Lean_Elab_Tactic_instToSnapshotTreeTacticFinishedSnapshot___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_saveState___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___lambda__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__1; static lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1___closed__1; LEAN_EXPORT uint8_t l_Lean_Elab_Term_withoutTacticIncrementality___rarg___lambda__1(uint8_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_applyVisibility___at_Lean_Elab_Term_expandDeclId___spec__5(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -897,8 +898,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_liftLevelM___rarg___boxed(lean_object* LEAN_EXPORT lean_object* l_Lean_Elab_withSaveInfoContext___at___private_Lean_Elab_Term_0__Lean_Elab_Term_withoutModifyingStateWithInfoAndMessagesImpl___spec__1(lean_object*); lean_object* l_Lean_RBNode_insert___at_Lean_MVarIdMap_insert___spec__1___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_findSomeRevMAux___at_Lean_Elab_Term_resolveLocalName___spec__9___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__6; -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoLeaf___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_instMonadTermElabM___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -912,6 +911,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_dropTermPa static lean_object* l_Lean_Elab_Term_withRestoreOrSaveFull___rarg___closed__12; lean_object* lean_io_mono_nanos_now(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_findSomeRevM_x3f___at_Lean_Elab_Term_resolveLocalName___spec__7___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19797_(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabUsingElabFns(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Term_LevelMVarErrorInfo_logError___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -939,7 +939,7 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_tryPostponeIfHasM LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabUsingElabFns___closed__2; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__2___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20103_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Option_set___at_Lean_Elab_Term_withoutMacroStackAtErr___spec__1(lean_object*, lean_object*, uint8_t); uint64_t l_Lean_Expr_hash(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -950,7 +950,6 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_expandDecl uint8_t l_Lean_BinderInfo_isInstImplicit(uint8_t); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_withDeclName___spec__13(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkAnnotation(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_withLogging___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_instToStringSyntheticMVarKind(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_synthesizeInstMVarCore___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -992,6 +991,8 @@ lean_object* l_Lean_RBNode_insert___at_Lean_FVarIdMap_insert___spec__1___rarg(le LEAN_EXPORT lean_object* l_Lean_Elab_isIncrementalElab___rarg___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_decorateErrorMessageWithLambdaImplicitVars___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_name_eq(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__4; +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__7; LEAN_EXPORT lean_object* l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at___private_Lean_Elab_Term_0__Lean_Elab_Term_withoutModifyingStateWithInfoAndMessagesImpl___spec__2(lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__24(lean_object*, lean_object*, size_t, size_t); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___lambda__3___closed__2; @@ -1009,12 +1010,14 @@ extern lean_object* l_Lean_warningAsError; static lean_object* l_Lean_Elab_Term_tryPostponeIfHasMVars___closed__1; extern lean_object* l_Lean_Elab_pp_macroStack; static lean_object* l_Lean_Elab_Term_mkConst___lambda__1___closed__2; +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Term_instMonadTermElabM___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Elab_Term_0__Lean_Elab_Term_isNoImplicitLambda(lean_object*); static lean_object* l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__10; LEAN_EXPORT lean_object* l_Lean_Elab_Term_isSaveInfoAnnotation_x3f___boxed(lean_object*); lean_object* l_Lean_Syntax_node2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__1; static lean_object* l_Lean_Elab_Term_TermElabM_toIO___rarg___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_mkConstWithLevelParams___at_Lean_Elab_Term_expandDeclId___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___lambda__1(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1059,6 +1062,7 @@ extern lean_object* l_Lean_diagnostics; uint8_t l_Lean_Syntax_isIdent(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabImplicitLambdaAux(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__10; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_resolveId_x3f___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_postponeElabTerm(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__46___boxed(lean_object*, lean_object*); @@ -1066,6 +1070,7 @@ lean_object* l_Lean_LocalDecl_fvarId(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isTacticBlock___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_logAt___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__2___lambda__2___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_postponeElabTerm___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771_(lean_object*); extern lean_object* l_Lean_Elab_abortTermExceptionId; LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_ensureType___spec__1___rarg(lean_object*); static lean_object* l_Lean_Elab_Term_resolveId_x3f___lambda__2___closed__3; @@ -1074,9 +1079,8 @@ LEAN_EXPORT lean_object* l_Lean_Elab_applyVisibility___at_Lean_Elab_Term_expandD LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutMacroStackAtErr(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkTacticMVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_withoutErrToSorry___rarg___closed__1; +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__3; static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Term_exposeLevelMVars___spec__7___rarg___closed__4; -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__2; -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__12; uint8_t l_Lean_LocalDecl_isAuxDecl(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_resolveLocalName_go___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_resolveGlobalName___at_Lean_Elab_Term_resolveLocalName_loop___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1109,16 +1113,15 @@ LEAN_EXPORT uint8_t l___private_Lean_Elab_Term_0__Lean_Elab_Term_isTacticBlock(l LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__34(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_exprToSyntax___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_containsPendingMVar___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3___closed__2; static lean_object* l_Lean_withTraceNode___at_Lean_Elab_Term_mkCoe___spec__1___lambda__3___closed__2; uint8_t l_Lean_PersistentHashMap_contains___at_Lean_MVarId_isAssigned___spec__1(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__7; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__4___lambda__1(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_instToSnapshotTreeTacticParsedSnapshot_go___spec__1___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_resolveName_process___closed__3; static lean_object* l_Lean_logAt___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__2___lambda__2___closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_MVarId_assign___at_Lean_Elab_Term_exprToSyntax___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__4; static lean_object* l_Lean_Elab_Term_throwErrorIfErrors___closed__2; LEAN_EXPORT lean_object* l_Lean_addDocString_x27___at_Lean_Elab_Term_expandDeclId___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_resolveName_process___closed__1; @@ -1131,7 +1134,6 @@ LEAN_EXPORT uint8_t l_Lean_PersistentArray_anyMAux___at_Lean_Elab_Term_addAutoBo uint8_t l_Lean_Environment_contains(lean_object*, lean_object*); static size_t l_Lean_Elab_Term_instInhabitedMVarErrorKind___closed__5; static lean_object* l_List_forIn_loop___at_Lean_Elab_Term_logUnassignedLevelMVarsUsingErrorInfos___spec__4___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627_(lean_object*); extern lean_object* l_Lean_inheritedTraceOptions; LEAN_EXPORT lean_object* l_Lean_Elab_isIncrementalElab___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Term_exposeLevelMVars___spec__7(lean_object*); @@ -1142,6 +1144,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Term_expandDeclId static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Term_exposeLevelMVars___spec__7___rarg___closed__2; LEAN_EXPORT lean_object* l_Lean_profileitM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__11(lean_object*); lean_object* l_Lean_Option_register___at_Lean_Elab_initFn____x40_Lean_Elab_AutoBound___hyg_6____spec__1(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_addAutoBoundImplicits_go(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at_Lean_Elab_Term_resolveLocalName___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isTypeAscription___closed__1; @@ -1164,7 +1167,9 @@ static lean_object* l_Lean_logAt___at_Lean_Elab_Term_MVarErrorInfo_logError___sp LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_withDeclName___spec__12(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withAutoBoundImplicit___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___closed__1; +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkConst___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__8; static lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError___closed__2; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_throwTypeMismatchError___spec__1(lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isHole___closed__1; @@ -1177,7 +1182,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_ensureHasType(lean_object*, lean_objec lean_object* l_Lean_LocalDecl_userName(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_addTermInfo___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isTacticBlock___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapMAux___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError_appendExtra(lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_setElabConfig(lean_object*); @@ -1185,6 +1189,7 @@ static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_decorateErrorMe LEAN_EXPORT lean_object* l_Lean_log___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerMVarErrorHoleInfo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_exposeLevelMVars(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__5; static lean_object* l_Lean_Elab_Tactic_instInhabitedTacticFinishedSnapshot___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkTermElabAttributeUnsafe(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortCommand___at_Lean_Elab_Term_ensureNoUnassignedMVars___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1194,6 +1199,7 @@ static lean_object* l_Lean_Elab_Term_instMonadBacktrackSavedStateTermElabM___clo extern lean_object* l_Lean_Linter_deprecatedAttr; LEAN_EXPORT lean_object* l_Lean_Elab_Term_instMonadMacroAdapterTermElabM___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Core_interruptExceptionId; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_checkDeprecated___at_Lean_Elab_Term_mkConst___spec__3___closed__9; LEAN_EXPORT lean_object* l_Lean_Elab_Term_isSaveInfoAnnotation_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_throwMVarError___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1201,6 +1207,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Term_expandDeclId LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at_Lean_Elab_Term_resolveLocalName___spec__8(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_withoutTacticIncrementality___rarg___lambda__3___closed__1; static lean_object* l_Lean_Elab_Term_resolveName___closed__4; +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__7; LEAN_EXPORT lean_object* l_Lean_Elab_Term_addTermInfo_x27(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_mkAuxName___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1212,7 +1219,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_throwTypeMismatchError(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkCoe___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshIdent___rarg___lambda__1(lean_object*, lean_object*, uint8_t, lean_object*); static lean_object* l_Lean_Elab_Term_mkCoe___closed__1; -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__3; +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__6; lean_object* l_Lean_instAddErrorMessageContextOfAddMessageContextOfMonad___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at_Lean_Elab_Term_resolveLocalName___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_PersistentArray_anyMAux___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__22(lean_object*, lean_object*); @@ -1222,7 +1229,6 @@ static lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError___lambda__1___closed static double l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2___closed__1; static lean_object* l_Lean_withTraceNode___at_Lean_Elab_Term_mkCoe___spec__1___lambda__4___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Term_universeConstraintsCheckpoint___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19758_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_instMonadMacroAdapterTermElabM___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Name_hasMacroScopes(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isNoImplicitLambda___boxed(lean_object*); @@ -1248,7 +1254,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_instMonadTermElabM___lambda__1___boxed static lean_object* l_Lean_Elab_Term_exprToSyntax___lambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapM___at_Lean_Elab_Term_withDeclName___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_collectUnassignedMVars(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__11; uint8_t l_Lean_Name_isAtomic(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_instInhabitedTermElabM___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1324,10 +1329,10 @@ static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Term_exposeLevelMVa static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_expandDeclId___spec__4___closed__4; lean_object* l_Lean_ParametricAttribute_getParam_x3f___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_CommandContextInfo_save___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_saveState___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_indentExpr(lean_object*); LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Term_mkCoe___spec__1___lambda__2___boxed(lean_object**); -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_BinderInfo_isExplicit(uint8_t); static lean_object* l_Lean_Elab_Term_withRestoreOrSaveFull___rarg___closed__7; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instInhabitedTacticFinishedSnapshot; @@ -1336,6 +1341,7 @@ static lean_object* l_Lean_Linter_checkDeprecated___at_Lean_Elab_Term_mkConst___ static lean_object* l_Lean_Elab_Term_exposeLevelMVars___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__14(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_isLetRecAuxMVar___lambda__3___closed__1; +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__5; LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitMain___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__3___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_isLetRecAuxMVar___closed__1; @@ -1367,10 +1373,9 @@ static lean_object* l_Lean_Elab_Term_withRestoreOrSaveFull___rarg___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_instInhabitedMVarErrorInfo; LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isExplicit___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__13___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Term_expandDeclId___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__4; -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__10; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Term_logUnassignedLevelMVarsUsingErrorInfos___spec__4___lambda__1(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_mkCoe___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_getDelayedMVarRoot___at_Lean_Elab_Term_isLetRecAuxMVar___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1406,7 +1411,6 @@ LEAN_EXPORT uint8_t l___private_Lean_Elab_Term_0__Lean_Elab_Term_isTypeAscriptio static lean_object* l_Lean_Elab_Term_exprToSyntax___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Term_exposeLevelMVars___spec__7___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutTacticIncrementality___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__3; static lean_object* l_Lean_Elab_Term_throwTypeMismatchError___rarg___closed__1; lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_CollectLevelMVars_visitExpr___spec__2(lean_object*); static lean_object* l_Lean_Elab_Term_withoutTacticIncrementality___rarg___lambda__3___closed__3; @@ -1432,6 +1436,7 @@ lean_object* lean_nat_mul(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_withDeclName___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerLevelMVarErrorExprInfo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Core_resetMessageLog(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__2; static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Term_exposeLevelMVars___spec__7___rarg___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Term_tryPostponeIfHasMVars(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortCommand___at_Lean_Elab_Term_ensureNoUnassignedMVars___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1454,6 +1459,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_resolveName___lambda__2___boxed(lean_o LEAN_EXPORT lean_object* l_Lean_Elab_Term_checkDeprecated___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_tryPostponeIfHasMVars_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_tryPostponeIfHasMVars___closed__5; +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Elab_Term_ContainsPendingMVar_visit___spec__2___boxed(lean_object*, lean_object*); uint8_t l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_visit___spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withInfoContext_x27(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1499,6 +1505,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkCoe(lean_object*, lean_object*, lean static lean_object* l_Lean_Elab_Term_tryPostponeIfHasMVars___closed__6; lean_object* l_Lean_registerBuiltinAttribute(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwPostpone___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_incrementalAttr; LEAN_EXPORT lean_object* l_Lean_Elab_Term_saveState___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_useImplicitLambda___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1507,7 +1514,6 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_resolveName_x27__ static lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Term_expandDeclId___spec__2___closed__1; static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isNoImplicitLambda___closed__1; static lean_object* l_Lean_Elab_applyVisibility___at_Lean_Elab_Term_expandDeclId___spec__5___closed__4; -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811_(lean_object*); lean_object* l_List_reverse___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_withInfoTreeContext___at_Lean_Elab_Term_withMacroExpansion___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withAuxDecl___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1519,19 +1525,20 @@ lean_object* l___private_Lean_ToExpr_0__Lean_Name_toExprAux(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerLevelMVarErrorInfo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withNarrowedArgTacticReuse___rarg___lambda__1(lean_object*, lean_object*); lean_object* l___private_Lean_MonadEnv_0__Lean_mkAuxNameAux(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instBEqCacheKey; static lean_object* l_List_foldl___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__2___closed__1; static lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Term_instMonadParentDeclTermElabM; static lean_object* l_Lean_Elab_Term_extraMsgToMsg___closed__1; size_t lean_usize_sub(size_t, size_t); +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_mk(lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__47(lean_object*, lean_object*, size_t, size_t); lean_object* l_Lean_PersistentArray_get_x21___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__9; LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isTypeAscription___lambda__1___boxed(lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__15(lean_object*, lean_object*, size_t, size_t); +LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666_(lean_object*); static lean_object* l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_throwMVarError___spec__2___rarg___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_observing___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_find___at_Lean_Elab_Term_MVarErrorInfo_logError_addArgName___spec__1___boxed(lean_object*, lean_object*); @@ -1567,7 +1574,6 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_addAutoBoundImpli uint8_t l_Lean_Expr_hasFVar(lean_object*); static lean_object* l_Lean_Elab_Term_withRestoreOrSaveFull___rarg___closed__8; static lean_object* l_Lean_Elab_isIncrementalElab___rarg___lambda__3___closed__1; -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__9; LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitMain___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__11(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_withRestoreOrSaveFull___rarg___closed__6; static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isTypeAscription___closed__4; @@ -1576,16 +1582,13 @@ LEAN_EXPORT lean_object* l_Lean_logAt___at___private_Lean_Elab_Term_0__Lean_Elab static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___lambda__7___closed__1; lean_object* l_Lean_MessageLog_append(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Term_withAutoBoundImplicit_loop___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__8; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instInhabitedTacticParsedSnapshotData(lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__2(lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Elab_Term_resolveName___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Level_isMVar(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__4___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withLevelNames___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_mkExplicitBinder___closed__2; -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__1; LEAN_EXPORT uint8_t l___private_Lean_Elab_Term_0__Lean_Elab_Term_isExplicitApp(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_throwMVarError___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_resolveName_x27___closed__2; @@ -1598,6 +1601,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_addTermInfo(lean_object*, lean_object* static lean_object* l_Lean_Core_transform___at_Lean_Elab_Term_exposeLevelMVars___spec__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_extraMsgToMsg(lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_postponeElabTermCore___closed__1; +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__2; extern lean_object* l_Lean_trace_profiler; LEAN_EXPORT lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Term_expandDeclId___spec__2___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutErrToSorry___rarg(lean_object*, lean_object*); @@ -1633,7 +1637,6 @@ LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBound lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallTelescopeReducingAux___rarg(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_localDeclDependsOn___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_withRestoreOrSaveFull___rarg___closed__17; -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__14; extern lean_object* l_Lean_KVMap_empty; LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapMAux___at_Lean_Elab_Term_withDeclName___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -1691,7 +1694,6 @@ LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapM___at_Lean_Elab_Term_without uint8_t lean_usize_dec_lt(size_t, size_t); static lean_object* l_Lean_Elab_Term_exposeLevelMVars___lambda__1___closed__1; lean_object* l_Lean_RBNode_find___at_Lean_NameMap_find_x3f___spec__1___rarg(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withAuxDecl___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at_Lean_Elab_Term_resolveLocalName___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_findSomeRevMAux___at_Lean_Elab_Term_resolveLocalName___spec__9(lean_object*, lean_object*); @@ -1701,22 +1703,24 @@ LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at_Lean_Elab_Term_resol LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__13(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Term_expandDeclId___spec__2___closed__4; +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___closed__2; lean_object* l_Lean_getExprMVarAssignment_x3f___at___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitMain___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_getResetInfoTrees___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__5___rarg___boxed(lean_object*, lean_object*); lean_object* l_Lean_Meta_mkLambdaFVars(lean_object*, lean_object*, uint8_t, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_realizeGlobalName(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_withoutModifyingStateWithInfoAndMessagesImpl___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20103____closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withAutoBoundImplicitForbiddenPred___rarg___lambda__1(lean_object*, lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__13; static lean_object* l_Lean_Elab_Term_instToStringSyntheticMVarKind___closed__1; static lean_object* l_Lean_Elab_Term_getInfoTreeWithContext_x3f___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_withMacroExpansionInfo___at_Lean_Elab_Term_withMacroExpansion___spec__1(lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___lambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Term_instInhabitedMVarErrorKind; LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Term_withAutoBoundImplicit_loop___spec__1(lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__15; LEAN_EXPORT lean_object* l_Lean_Elab_Term_observing(lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__1; uint8_t l_Lean_Exception_isRuntime(lean_object*); lean_object* l_Lean_Expr_lam___override(lean_object*, lean_object*, lean_object*, uint8_t); static lean_object* l_Lean_Elab_Term_exposeLevelMVars___lambda__2___closed__5; @@ -1730,7 +1734,6 @@ LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_v LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoLeaf___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_mkConsts___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withNarrowedArgTacticReuse___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoTree___at_Lean_Elab_Term_addDotCompletionInfo___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isTacticBlock___closed__3; static lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError___lambda__1___closed__6; @@ -1741,7 +1744,6 @@ uint8_t l_Lean_Expr_isFVar(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_exprToSyntax___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at_Lean_Elab_Term_withDeclName___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_SavedState_restore___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__3; static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___lambda__7___closed__2; static lean_object* l_Lean_Elab_Term_expandDeclId___closed__2; static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabUsingElabFns___closed__1; @@ -1758,17 +1760,19 @@ lean_object* l_Lean_getStructureFieldsFlattened(lean_object*, lean_object*, uint lean_object* l_Lean_Expr_mvarId_x21(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabImplicitLambda_loop___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwPostpone___at_Lean_Elab_Term_tryPostpone___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_addDocString_x27___at_Lean_Elab_Term_expandDeclId___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_instInhabitedState___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_throwMVarError___spec__2___rarg(lean_object*); uint8_t l_Lean_Elab_isValidAutoBoundImplicitName(lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Core_withIncRecDepth___at_Lean_Elab_Term_exposeLevelMVars___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_throwError___at_Lean_Attribute_Builtin_ensureNoArgs___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__6; LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__10___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_throwAutoBoundImplicitLocal___at_Lean_Elab_Term_resolveName_process___spec__1___closed__2; lean_object* l_String_toSubstring_x27(lean_object*); LEAN_EXPORT lean_object* l_Lean_getDelayedMVarAssignment_x3f___at_Lean_Elab_Term_ContainsPendingMVar_visit___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__8; static lean_object* l_Lean_Elab_Term_synthesizeInstMVarCore___lambda__3___closed__4; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__9(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_mkCoe___lambda__2___closed__2; @@ -1793,6 +1797,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_tryPostpone(lean_object*, lean_object* lean_object* l_List_filterTR_loop___at_Lean_filterFieldList___spec__1(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_PersistentArray_anyMAux___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__38(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at_Lean_Elab_Term_resolveLocalName___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); uint8_t l___private_Lean_Message_0__Lean_beqMessageSeverity____x40_Lean_Message___hyg_106_(uint8_t, uint8_t); LEAN_EXPORT lean_object* l_Lean_Elab_Term_removeSaveInfoAnnotation(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Term_0__Lean_Elab_Term_withoutModifyingStateWithInfoAndMessagesImpl___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1800,13 +1805,11 @@ static lean_object* l_Lean_Elab_Term_exprToSyntax___lambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Term_getLetRecsToLift___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutTacticReuse___rarg___lambda__1(uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__10___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__5; static lean_object* l_Lean_addDocString___at_Lean_Elab_Term_expandDeclId___spec__9___closed__2; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Term_0__Lean_Elab_Term_withoutModifyingStateWithInfoAndMessagesImpl___spec__7(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerLevelMVarErrorExprInfo___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Term_expandDeclId___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20064_(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_expandDeclId___spec__4___closed__5; static lean_object* l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__8; static lean_object* l_Lean_Elab_Term_mkExplicitBinder___closed__8; @@ -1830,8 +1833,8 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_debug_byAsSorry; static lean_object* l_Lean_Elab_Tactic_instToSnapshotTreeTacticParsedSnapshot_go___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_useImplicitLambda___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withAutoBoundImplicit_loop___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__5; static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isLambdaWithImplicit___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617_(lean_object*); static lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError___lambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_throwTypeMismatchError___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_contains___at_Lean_Elab_Term_logUnassignedLevelMVarsUsingErrorInfos___spec__1(lean_object*, lean_object*); @@ -1840,7 +1843,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutTacticReuse___rarg___lambda__2( LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Term_mkCoe___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); double lean_float_sub(double, double); LEAN_EXPORT lean_object* l_Lean_Elab_Term_ContainsPendingMVar_visit___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578_(lean_object*); LEAN_EXPORT lean_object* l_Lean_logAt___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_hasExprMVar(lean_object*); lean_object* l_Lean_Meta_processPostponed(uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -34168,15 +34170,7 @@ return x_22; } } } -static lean_object* _init_l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("attribute application", 21, 21); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___boxed__const__1() { +static lean_object* _init_l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___lambda__2___boxed__const__1() { _start: { size_t x_1; lean_object* x_2; @@ -34185,6 +34179,32 @@ x_2 = lean_box_usize(x_1); return x_2; } } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +size_t x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_12 = lean_array_size(x_1); +x_13 = lean_box_usize(x_12); +x_14 = l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___lambda__2___boxed__const__1; +lean_inc(x_2); +x_15 = lean_alloc_closure((void*)(l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___lambda__1___boxed), 12, 5); +lean_closure_set(x_15, 0, x_2); +lean_closure_set(x_15, 1, x_3); +lean_closure_set(x_15, 2, x_1); +lean_closure_set(x_15, 3, x_13); +lean_closure_set(x_15, 4, x_14); +x_16 = l_Lean_Elab_Term_withDeclName___rarg(x_2, x_15, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_16; +} +} +static lean_object* _init_l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("attribute application", 21, 21); +return x_1; +} +} LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { @@ -34195,34 +34215,31 @@ x_12 = lean_box(0); x_13 = lean_name_eq(x_1, x_12); if (x_13 == 0) { -size_t x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_14 = lean_array_size(x_2); -x_15 = lean_box_usize(x_14); -x_16 = l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___boxed__const__1; -x_17 = lean_alloc_closure((void*)(l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___lambda__1___boxed), 12, 5); -lean_closure_set(x_17, 0, x_1); -lean_closure_set(x_17, 1, x_3); -lean_closure_set(x_17, 2, x_2); -lean_closure_set(x_17, 3, x_15); -lean_closure_set(x_17, 4, x_16); -x_18 = l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___closed__1; -x_19 = l_Lean_profileitM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__11___rarg(x_18, x_11, x_17, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_14 = lean_box(0); +x_15 = lean_alloc_closure((void*)(l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___lambda__2___boxed), 11, 4); +lean_closure_set(x_15, 0, x_2); +lean_closure_set(x_15, 1, x_1); +lean_closure_set(x_15, 2, x_3); +lean_closure_set(x_15, 3, x_14); +x_16 = l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___closed__1; +x_17 = l_Lean_profileitM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__11___rarg(x_16, x_11, x_15, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_11); -return x_19; +return x_17; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_20 = lean_box(0); -x_21 = lean_alloc_closure((void*)(l_ReaderT_pure___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__12___rarg___boxed), 8, 1); -lean_closure_set(x_21, 0, x_20); -x_22 = l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___closed__1; -x_23 = l_Lean_profileitM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__11___rarg(x_22, x_11, x_21, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_18 = lean_box(0); +x_19 = lean_alloc_closure((void*)(l_ReaderT_pure___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__12___rarg___boxed), 8, 1); +lean_closure_set(x_19, 0, x_18); +x_20 = l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___closed__1; +x_21 = l_Lean_profileitM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__11___rarg(x_20, x_11, x_19, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_11); -return x_23; +return x_21; } } } @@ -34415,6 +34432,15 @@ lean_dec(x_3); return x_15; } } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +x_12 = l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_4); +return x_12; +} +} LEAN_EXPORT lean_object* l_Lean_Elab_Term_applyAttributesAt(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { @@ -45448,7 +45474,7 @@ lean_dec(x_1); return x_9; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__1() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__1() { _start: { lean_object* x_1; @@ -45456,7 +45482,7 @@ x_1 = lean_mk_string_unchecked("debug", 5, 5); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__2() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__2() { _start: { lean_object* x_1; @@ -45464,17 +45490,17 @@ x_1 = lean_mk_string_unchecked("byAsSorry", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__3() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__1; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__2; +x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__1; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__2; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__4() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__4() { _start: { lean_object* x_1; @@ -45482,13 +45508,13 @@ x_1 = lean_mk_string_unchecked("replace `by ..` blocks with `sorry` IF the expec return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__5() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__5() { _start: { uint8_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = 0; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__1; -x_3 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__4; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__1; +x_3 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__4; x_4 = lean_box(x_1); x_5 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_5, 0, x_4); @@ -45497,26 +45523,26 @@ lean_ctor_set(x_5, 2, x_3); return x_5; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__6() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__5; x_2 = l_Lean_Elab_Term_withoutTacticIncrementality___rarg___lambda__3___closed__2; x_3 = l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__7; -x_4 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__1; -x_5 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__2; +x_4 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__1; +x_5 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__2; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__3; -x_3 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__5; -x_4 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__6; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__3; +x_3 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__5; +x_4 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__6; x_5 = l_Lean_Option_register___at_Lean_Elab_initFn____x40_Lean_Elab_AutoBound___hyg_6____spec__1(x_2, x_3, x_4, x_1); return x_5; } @@ -68129,7 +68155,7 @@ lean_dec(x_3); return x_9; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__1() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__1() { _start: { lean_object* x_1; @@ -68137,17 +68163,17 @@ x_1 = lean_mk_string_unchecked("letrec", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__2() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Elab_Term_withoutTacticIncrementality___rarg___lambda__3___closed__2; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__1; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__1; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__3() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -68157,27 +68183,27 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__4() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__3; +x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__3; x_2 = l_Lean_Elab_Term_withoutTacticIncrementality___rarg___lambda__3___closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__5() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__4; +x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__4; x_2 = l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__7; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__6() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__6() { _start: { lean_object* x_1; @@ -68185,17 +68211,17 @@ x_1 = lean_mk_string_unchecked("initFn", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__7() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__5; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__6; +x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__5; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__8() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__8() { _start: { lean_object* x_1; @@ -68203,47 +68229,47 @@ x_1 = lean_mk_string_unchecked("_@", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__9() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__7; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__8; +x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__7; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__8; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__10() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__9; +x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__9; x_2 = l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__5; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__11() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__10; +x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__10; x_2 = l_Lean_Elab_Term_withoutTacticIncrementality___rarg___lambda__3___closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__12() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__11; +x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__11; x_2 = l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__7; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__13() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__13() { _start: { lean_object* x_1; @@ -68251,33 +68277,33 @@ x_1 = lean_mk_string_unchecked("_hyg", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__14() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__12; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__13; +x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__12; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__13; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__15() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__14; -x_2 = lean_unsigned_to_nat(17274u); +x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__14; +x_2 = lean_unsigned_to_nat(17313u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313_(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__2; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__2; x_3 = 0; -x_4 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__15; +x_4 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__15; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); return x_5; } @@ -68684,7 +68710,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_isLetRecAuxMVar(lean_object* x_1, lean _start: { lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_9 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__2; +x_9 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__2; x_10 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_9, x_2, x_3, x_4, x_5, x_6, x_7, x_8); x_11 = lean_ctor_get(x_10, 0); lean_inc(x_11); @@ -76094,7 +76120,7 @@ lean_object* x_14; uint8_t x_15; lean_object* x_16; x_14 = lean_ctor_get(x_13, 1); lean_inc(x_14); lean_dec(x_13); -x_15 = lean_ctor_get_uint8(x_2, sizeof(void*)*2); +x_15 = lean_ctor_get_uint8(x_2, sizeof(void*)*3); lean_inc(x_6); x_16 = l_Lean_Elab_applyVisibility___at_Lean_Elab_Term_expandDeclId___spec__5(x_15, x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_14); if (lean_obj_tag(x_16) == 0) @@ -77154,7 +77180,7 @@ lean_inc(x_32); x_33 = lean_ctor_get(x_30, 1); lean_inc(x_33); lean_dec(x_30); -x_34 = lean_ctor_get(x_3, 0); +x_34 = lean_ctor_get(x_3, 1); lean_inc(x_34); lean_dec(x_3); lean_inc(x_32); @@ -78495,87 +78521,87 @@ x_3 = lean_alloc_closure((void*)(l_Lean_Elab_withoutModifyingStateWithInfoAndMes return x_3; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__1() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__4; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__6; +x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__4; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__2() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__1; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__8; +x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__1; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__8; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__3() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__2; +x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__2; x_2 = l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__5; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__4() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__3; +x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__3; x_2 = l_Lean_Elab_Term_withoutTacticIncrementality___rarg___lambda__3___closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__5() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__4; +x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__4; x_2 = l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__7; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__6() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__5; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__13; +x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__5; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__13; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__7() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__6; -x_2 = lean_unsigned_to_nat(19578u); +x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__6; +x_2 = lean_unsigned_to_nat(19617u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__8() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Elab_Term_withoutTacticIncrementality___rarg___lambda__3___closed__2; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__1; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__1; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__9() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -78585,13 +78611,13 @@ x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617_(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; x_2 = l___private_Lean_Elab_Term_0__Lean_Elab_Term_postponeElabTermCore___closed__2; x_3 = 0; -x_4 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__7; +x_4 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__7; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); if (lean_obj_tag(x_5) == 0) { @@ -78607,7 +78633,7 @@ lean_object* x_9; lean_object* x_10; lean_object* x_11; x_9 = lean_ctor_get(x_8, 1); lean_inc(x_9); lean_dec(x_8); -x_10 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__8; +x_10 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__8; x_11 = l_Lean_registerTraceClass(x_10, x_3, x_4, x_9); if (lean_obj_tag(x_11) == 0) { @@ -78615,7 +78641,7 @@ lean_object* x_12; lean_object* x_13; lean_object* x_14; x_12 = lean_ctor_get(x_11, 1); lean_inc(x_12); lean_dec(x_11); -x_13 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__9; +x_13 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__9; x_14 = l_Lean_registerTraceClass(x_13, x_3, x_4, x_12); return x_14; } @@ -78689,7 +78715,7 @@ return x_26; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; @@ -78700,7 +78726,7 @@ lean_ctor_set(x_6, 1, x_4); return x_6; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__1() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__1() { _start: { lean_object* x_1; @@ -78708,17 +78734,17 @@ x_1 = lean_mk_string_unchecked("incremental", 11, 11); return x_1; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__2() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__1; +x_2 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__3() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__3() { _start: { lean_object* x_1; @@ -78726,18 +78752,18 @@ x_1 = lean_mk_string_unchecked("incrementalAttr", 15, 15); return x_1; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__4() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__5; x_2 = l_Lean_Elab_Term_withoutTacticIncrementality___rarg___lambda__3___closed__2; -x_3 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__3; +x_3 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__3; x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__5() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__5() { _start: { lean_object* x_1; @@ -78745,39 +78771,39 @@ x_1 = lean_mk_string_unchecked("Marks an elaborator (tactic or command, currentl return x_1; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__6() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__6() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____lambda__1___boxed), 4, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____lambda__1___boxed), 4, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; uint8_t x_6; lean_object* x_7; -x_2 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__2; -x_3 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__5; -x_4 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__6; -x_5 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__4; +x_2 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__2; +x_3 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__5; +x_4 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__6; +x_5 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__4; x_6 = 0; x_7 = l_Lean_registerTagAttribute(x_2, x_3, x_4, x_5, x_6, x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____lambda__1(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____lambda__1(x_1, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19758_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19797_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; uint8_t x_4; @@ -78845,7 +78871,7 @@ return x_13; } } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___closed__1() { _start: { lean_object* x_1; @@ -78853,40 +78879,40 @@ x_1 = lean_mk_string_unchecked("addBuiltinIncrementalElab", 25, 25); return x_1; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__2() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__5; x_2 = l_Lean_Elab_Term_withoutTacticIncrementality___rarg___lambda__3___closed__2; -x_3 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__1; +x_3 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___closed__1; x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__3() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__2; +x_2 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___closed__2; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_inc(x_1); x_6 = l___private_Lean_ToExpr_0__Lean_Name_toExprAux(x_1); -x_7 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__3; +x_7 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___closed__3; x_8 = l_Lean_Expr_app___override(x_7, x_6); x_9 = l_Lean_declareBuiltin(x_1, x_8, x_3, x_4, x_5); return x_9; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__2___closed__1() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__2___closed__1() { _start: { lean_object* x_1; @@ -78894,16 +78920,16 @@ x_1 = lean_mk_string_unchecked("invalid attribute 'builtin_incremental', must be return x_1; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__2___closed__2() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__2___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__2___closed__1; +x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__2___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__2(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__2(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; @@ -78921,7 +78947,7 @@ if (x_10 == 0) { lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_dec(x_1); -x_11 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__2___closed__2; +x_11 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__2___closed__2; x_12 = l_Lean_throwError___at_Lean_registerTagAttribute___spec__1(x_11, x_4, x_5, x_8); lean_dec(x_4); x_13 = !lean_is_exclusive(x_12); @@ -78947,7 +78973,7 @@ else { lean_object* x_17; lean_object* x_18; x_17 = lean_box(0); -x_18 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1(x_1, x_17, x_4, x_5, x_8); +x_18 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1(x_1, x_17, x_4, x_5, x_8); lean_dec(x_4); return x_18; } @@ -78978,7 +79004,7 @@ return x_22; } } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3___closed__1() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3___closed__1() { _start: { lean_object* x_1; @@ -78986,35 +79012,35 @@ x_1 = lean_mk_string_unchecked("attribute cannot be erased", 26, 26); return x_1; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3___closed__2() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3___closed__1; +x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; -x_5 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3___closed__2; +x_5 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3___closed__2; x_6 = l_Lean_throwError___at_Lean_Attribute_Builtin_ensureNoArgs___spec__2(x_5, x_2, x_3, x_4); return x_6; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__1() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__6; -x_2 = lean_unsigned_to_nat(19811u); +x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__6; +x_2 = lean_unsigned_to_nat(19850u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__2() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__2() { _start: { lean_object* x_1; @@ -79022,17 +79048,17 @@ x_1 = lean_mk_string_unchecked("builtin_incremental", 19, 19); return x_1; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__3() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__2; +x_2 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__4() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__4() { _start: { lean_object* x_1; @@ -79040,7 +79066,7 @@ x_1 = lean_mk_string_unchecked("(builtin) ", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__5() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; @@ -79053,29 +79079,29 @@ lean_dec(x_2); x_4 = lean_ctor_get(x_3, 2); lean_inc(x_4); lean_dec(x_3); -x_5 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__4; +x_5 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__4; x_6 = lean_string_append(x_5, x_4); lean_dec(x_4); return x_6; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__6() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__5; +x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__5; x_2 = l_Lean_Elab_Term_extraMsgToMsg___closed__3; x_3 = lean_string_append(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__7() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; -x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__1; -x_2 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__3; -x_3 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__6; +x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__1; +x_2 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__3; +x_3 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__6; x_4 = 1; x_5 = lean_alloc_ctor(0, 3, 1); lean_ctor_set(x_5, 0, x_1); @@ -79085,29 +79111,29 @@ lean_ctor_set_uint8(x_5, sizeof(void*)*3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__8() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__8() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__2___boxed), 6, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__2___boxed), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__9() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__9() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3___boxed), 4, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3___boxed), 4, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__10() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__7; -x_2 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__8; -x_3 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__9; +x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__7; +x_2 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__8; +x_3 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__9; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -79115,42 +79141,42 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__10; +x_2 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__10; x_3 = l_Lean_registerBuiltinAttribute(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; -x_6 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1(x_1, x_2, x_3, x_4, x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { uint8_t x_7; lean_object* x_8; x_7 = lean_unbox(x_3); lean_dec(x_3); -x_8 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__2(x_1, x_2, x_7, x_4, x_5, x_6); +x_8 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__2(x_1, x_2, x_7, x_4, x_5, x_6); lean_dec(x_5); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3(x_1, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); @@ -79327,23 +79353,23 @@ x_7 = l_Lean_Elab_isIncrementalElab___rarg___lambda__4(x_1, x_2, x_3, x_4, x_6); return x_7; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20064____closed__1() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20103____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__6; -x_2 = lean_unsigned_to_nat(20064u); +x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__6; +x_2 = lean_unsigned_to_nat(20103u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20064_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20103_(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; x_2 = l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabImplicitLambdaAux___closed__2; x_3 = 0; -x_4 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20064____closed__1; +x_4 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20103____closed__1; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); return x_5; } @@ -79821,10 +79847,10 @@ l_Lean_Elab_logException___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAt lean_mark_persistent(l_Lean_Elab_logException___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__7___closed__2); l_Lean_Elab_logException___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__7___closed__3 = _init_l_Lean_Elab_logException___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__7___closed__3(); lean_mark_persistent(l_Lean_Elab_logException___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__7___closed__3); +l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___lambda__2___boxed__const__1 = _init_l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___lambda__2___boxed__const__1(); +lean_mark_persistent(l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___lambda__2___boxed__const__1); l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___closed__1 = _init_l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___closed__1(); lean_mark_persistent(l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___closed__1); -l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___boxed__const__1 = _init_l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___boxed__const__1(); -lean_mark_persistent(l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___boxed__const__1); l_Lean_Elab_Term_mkTypeMismatchError___closed__1 = _init_l_Lean_Elab_Term_mkTypeMismatchError___closed__1(); lean_mark_persistent(l_Lean_Elab_Term_mkTypeMismatchError___closed__1); l_Lean_Elab_Term_mkTypeMismatchError___closed__2 = _init_l_Lean_Elab_Term_mkTypeMismatchError___closed__2(); @@ -79929,19 +79955,19 @@ l___private_Lean_Elab_Term_0__Lean_Elab_Term_postponeElabTermCore___closed__4 = lean_mark_persistent(l___private_Lean_Elab_Term_0__Lean_Elab_Term_postponeElabTermCore___closed__4); l___private_Lean_Elab_Term_0__Lean_Elab_Term_postponeElabTermCore___closed__5 = _init_l___private_Lean_Elab_Term_0__Lean_Elab_Term_postponeElabTermCore___closed__5(); lean_mark_persistent(l___private_Lean_Elab_Term_0__Lean_Elab_Term_postponeElabTermCore___closed__5); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__1 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__1(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__1); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__2 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__2(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__2); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__3 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__3(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__3); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__4 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__4(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__4); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__5 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__5(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__5); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__6 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__6(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__6); -if (builtin) {res = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627_(lean_io_mk_world()); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__1 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__1(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__1); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__2 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__2(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__2); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__3 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__3(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__3); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__4 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__4(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__4); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__5 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__5(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__5); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__6 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__6(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__6); +if (builtin) {res = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_Elab_Term_debug_byAsSorry = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Elab_Term_debug_byAsSorry); @@ -80101,37 +80127,37 @@ l_Lean_Elab_Term_mkAuxName___closed__1 = _init_l_Lean_Elab_Term_mkAuxName___clos lean_mark_persistent(l_Lean_Elab_Term_mkAuxName___closed__1); l_Lean_Elab_Term_mkAuxName___closed__2 = _init_l_Lean_Elab_Term_mkAuxName___closed__2(); lean_mark_persistent(l_Lean_Elab_Term_mkAuxName___closed__2); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__1 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__1(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__1); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__2 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__2(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__2); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__3 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__3(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__3); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__4 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__4(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__4); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__5 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__5(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__5); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__6 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__6(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__6); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__7 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__7(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__7); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__8 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__8(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__8); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__9 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__9(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__9); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__10 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__10(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__10); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__11 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__11(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__11); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__12 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__12(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__12); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__13 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__13(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__13); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__14 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__14(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__14); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__15 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__15(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__15); -if (builtin) {res = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274_(lean_io_mk_world()); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__1 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__1(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__1); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__2 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__2(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__2); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__3 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__3(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__3); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__4 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__4(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__4); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__5 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__5(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__5); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__6 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__6(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__6); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__7 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__7(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__7); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__8 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__8(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__8); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__9 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__9(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__9); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__10 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__10(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__10); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__11 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__11(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__11); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__12 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__12(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__12); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__13 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__13(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__13); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__14 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__14(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__14); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__15 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__15(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__15); +if (builtin) {res = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l_Lean_Elab_Term_isLetRecAuxMVar___lambda__3___closed__1 = _init_l_Lean_Elab_Term_isLetRecAuxMVar___lambda__3___closed__1(); @@ -80290,95 +80316,95 @@ l_Lean_Elab_Term_exprToSyntax___lambda__1___closed__3 = _init_l_Lean_Elab_Term_e lean_mark_persistent(l_Lean_Elab_Term_exprToSyntax___lambda__1___closed__3); l_Lean_Elab_Term_exprToSyntax___lambda__1___closed__4 = _init_l_Lean_Elab_Term_exprToSyntax___lambda__1___closed__4(); lean_mark_persistent(l_Lean_Elab_Term_exprToSyntax___lambda__1___closed__4); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__1 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__1(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__1); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__2 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__2(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__2); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__3 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__3(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__3); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__4 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__4(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__4); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__5 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__5(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__5); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__6 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__6(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__6); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__7 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__7(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__7); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__8 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__8(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__8); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__9 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__9(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__9); -if (builtin) {res = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578_(lean_io_mk_world()); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__1 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__1(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__1); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__2 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__2(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__2); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__3 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__3(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__3); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__4 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__4(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__4); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__5 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__5(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__5); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__6 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__6(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__6); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__7 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__7(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__7); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__8 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__8(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__8); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__9 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__9(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__9); +if (builtin) {res = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__1 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__1(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__1); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__2 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__2(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__2); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__3 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__3(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__3); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__4 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__4(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__4); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__5 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__5(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__5); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__6 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__6(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__6); -if (builtin) {res = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732_(lean_io_mk_world()); +}l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__1 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__1(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__1); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__2 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__2(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__2); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__3 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__3(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__3); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__4 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__4(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__4); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__5 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__5(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__5); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__6 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__6(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__6); +if (builtin) {res = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_Elab_incrementalAttr = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Elab_incrementalAttr); lean_dec_ref(res); -}if (builtin) {res = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19758_(lean_io_mk_world()); +}if (builtin) {res = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19797_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_Elab_builtinIncrementalElabs = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Elab_builtinIncrementalElabs); lean_dec_ref(res); }l_Lean_Elab_addBuiltinIncrementalElab___closed__1 = _init_l_Lean_Elab_addBuiltinIncrementalElab___closed__1(); lean_mark_persistent(l_Lean_Elab_addBuiltinIncrementalElab___closed__1); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__1 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__1); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__2 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__2); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__3 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__3); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__2___closed__1 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__2___closed__1(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__2___closed__1); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__2___closed__2 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__2___closed__2(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__2___closed__2); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3___closed__1 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3___closed__1(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3___closed__1); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3___closed__2 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3___closed__2(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3___closed__2); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__1 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__1(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__1); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__2 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__2(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__2); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__3 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__3(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__3); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__4 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__4(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__4); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__5 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__5(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__5); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__6 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__6(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__6); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__7 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__7(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__7); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__8 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__8(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__8); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__9 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__9(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__9); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__10 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__10(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__10); -if (builtin) {res = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811_(lean_io_mk_world()); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___closed__1 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___closed__1); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___closed__2 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___closed__2); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___closed__3 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___closed__3); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__2___closed__1 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__2___closed__1); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__2___closed__2 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__2___closed__2(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__2___closed__2); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3___closed__1 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3___closed__1); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3___closed__2 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3___closed__2(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3___closed__2); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__1 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__1(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__1); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__2 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__2(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__2); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__3 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__3(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__3); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__4 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__4(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__4); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__5 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__5(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__5); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__6 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__6(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__6); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__7 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__7(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__7); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__8 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__8(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__8); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__9 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__9(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__9); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__10 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__10(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__10); +if (builtin) {res = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l_Lean_Elab_isIncrementalElab___rarg___lambda__3___closed__1 = _init_l_Lean_Elab_isIncrementalElab___rarg___lambda__3___closed__1(); lean_mark_persistent(l_Lean_Elab_isIncrementalElab___rarg___lambda__3___closed__1); l_Lean_Elab_isIncrementalElab___rarg___closed__1 = _init_l_Lean_Elab_isIncrementalElab___rarg___closed__1(); lean_mark_persistent(l_Lean_Elab_isIncrementalElab___rarg___closed__1); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20064____closed__1 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20064____closed__1(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20064____closed__1); -if (builtin) {res = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20064_(lean_io_mk_world()); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20103____closed__1 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20103____closed__1(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20103____closed__1); +if (builtin) {res = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20103_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }return lean_io_result_mk_ok(lean_box(0)); diff --git a/stage0/stdlib/Lean/Language/Basic.c b/stage0/stdlib/Lean/Language/Basic.c index 36aad633d8d7..e42c30ce744c 100644 --- a/stage0/stdlib/Lean/Language/Basic.c +++ b/stage0/stdlib/Lean/Language/Basic.c @@ -24,7 +24,6 @@ LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Language_SnapshotTree_tr lean_object* l_Lean_Json_compress(lean_object*); extern lean_object* l_Lean_profiler; LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Language_SnapshotTree_trace_go___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__5; LEAN_EXPORT lean_object* l_Lean_Language_SnapshotTask_cancel___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Language_withAlwaysResolvedPromises___spec__2___rarg___lambda__1___boxed(lean_object*, lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); @@ -66,7 +65,6 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Language_reportMess LEAN_EXPORT lean_object* l_Lean_Language_SnapshotTask_ofIO(lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Language_instInhabitedDynamicSnapshot___spec__1(lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); -static lean_object* l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__3; static lean_object* l___auto____x40_Lean_Language_Basic___hyg_62____closed__40; LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_toTyped_x3f(lean_object*); static lean_object* l_Lean_Language_SnapshotTree_trace_go___lambda__2___closed__1; @@ -78,6 +76,7 @@ static lean_object* l___auto____x40_Lean_Language_Basic___hyg_62____closed__23; static lean_object* l_Lean_Language_reportMessages___closed__1; lean_object* l_Lean_Elab_InfoTree_format(lean_object*, lean_object*, lean_object*); uint8_t lean_float_decLt(double, double); +static lean_object* l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__4; static lean_object* l_Lean_Language_SnapshotTree_trace_go___closed__10; LEAN_EXPORT lean_object* l_Lean_Language_instToSnapshotTreeDynamicSnapshot(lean_object*); static lean_object* l_Lean_Language_SnapshotTree_trace_go___closed__6; @@ -104,7 +103,6 @@ lean_object* lean_string_utf8_byte_size(lean_object*); static lean_object* l_Lean_Language_SnapshotTree_trace_go___closed__7; LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Language_SnapshotTree_trace_go___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_withHeaderExceptions___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__1; static lean_object* l___auto____x40_Lean_Language_Basic___hyg_62____closed__20; lean_object* l_IO_Promise_resolve___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); @@ -124,6 +122,8 @@ LEAN_EXPORT lean_object* l_Lean_Language_SnapshotTree_runAndReport___boxed(lean_ static lean_object* l_Lean_Language_instInhabitedSnapshotTree___closed__1; static lean_object* l_Lean_Language_diagnosticsOfHeaderError___closed__1; LEAN_EXPORT lean_object* l_Lean_Language_SnapshotTree_trace_go___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__3; +LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___rarg___lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_SnapshotTask_pure(lean_object*); LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_Language_SnapshotTree_trace_go___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___auto____x40_Lean_Language_Basic___hyg_62____closed__21; @@ -161,6 +161,7 @@ lean_object* l_Lean_addMessageContextPartial___at_Lean_Core_instAddMessageContex LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Language_SnapshotTree_trace_go___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_SnapshotTree_forM___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Language_Snapshot_instInhabitedDiagnostics___closed__5; +static lean_object* l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__2; LEAN_EXPORT lean_object* l_Lean_Language_withAlwaysResolvedPromise___rarg___lambda__2___boxed(lean_object*); static lean_object* l___auto____x40_Lean_Language_Basic___hyg_62____closed__1; static lean_object* l_Lean_Language_instInhabitedDynamicSnapshot___closed__3; @@ -170,6 +171,7 @@ static lean_object* l_Lean_Language_instInhabitedDynamicSnapshot___closed__1; LEAN_EXPORT lean_object* l_Lean_PersistentArray_forMAux___at_Lean_Language_reportMessages___spec__3(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Language_SnapshotTree_trace_go___closed__5; LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Language_SnapshotTree_trace_go___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_thunk_get_own(lean_object*); static double l_Lean_withTraceNode___at_Lean_Language_SnapshotTree_trace_go___spec__5___lambda__4___closed__5; LEAN_EXPORT lean_object* l_Lean_MessageLog_forM___at_Lean_Language_reportMessages___spec__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___auto____x40_Lean_Language_Basic___hyg_62____closed__22; @@ -179,7 +181,6 @@ extern lean_object* l_Task_Priority_default; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Language_withAlwaysResolvedPromises___spec__2___rarg___lambda__2(lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_instInhabitedSnapshotTask___rarg(lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057_(lean_object*); static lean_object* l_Lean_Language_SnapshotTree_trace_go___closed__11; static lean_object* l_Lean_Language_Snapshot_instInhabitedDiagnostics___closed__1; extern lean_object* l_Lean_MessageLog_empty; @@ -207,6 +208,7 @@ static lean_object* l_Lean_Language_instInhabitedDynamicSnapshot___closed__4; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Language_reportMessages___spec__4(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_withAlwaysResolvedPromises___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_mkIncrementalProcessor___elambda__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_mk_thunk(lean_object*); LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Language_SnapshotTree_trace_go___spec__5___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Language_SnapshotTree_getAll___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*); lean_object* l___private_Lean_Util_Trace_0__Lean_addTraceNode___at_Lean_compileDecl___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -218,6 +220,7 @@ LEAN_EXPORT lean_object* l_Lean_Language_mkIncrementalProcessor___elambda__1(lea double l_Float_ofScientific(lean_object*, uint8_t, lean_object*); static lean_object* l_Lean_withTraceNode___at_Lean_Language_SnapshotTree_trace_go___spec__5___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Language_SnapshotTree_getAll___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__5; static lean_object* l___auto____x40_Lean_Language_Basic___hyg_62____closed__8; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Language_withAlwaysResolvedPromises___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Language_reportMessages___lambda__2___closed__1; @@ -225,6 +228,7 @@ LEAN_EXPORT lean_object* l_Functor_mapRev___at_Lean_Language_reportMessages___sp LEAN_EXPORT lean_object* l_Lean_MessageLog_forM___at_Lean_Language_reportMessages___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_instMonadLiftProcessingMProcessingTIO___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l___auto____x40_Lean_Language_Basic___hyg_62____closed__4; +LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Language_instInhabitedDynamicSnapshot___spec__1___lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Language_reportMessages___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Language_SnapshotTree_trace_go___spec__5___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Language_withAlwaysResolvedPromises___spec__2(lean_object*, lean_object*); @@ -238,7 +242,6 @@ lean_object* l_IO_println___at_Lean_Environment_displayStats___spec__3(lean_obje LEAN_EXPORT lean_object* l_Lean_Language_withAlwaysResolvedPromise(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Language_withHeaderExceptions___rarg___closed__1; static lean_object* l_Lean_Language_SnapshotTree_trace_go___lambda__3___closed__2; -static lean_object* l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__2; static lean_object* l___auto____x40_Lean_Language_Basic___hyg_62____closed__37; static lean_object* l___auto____x40_Lean_Language_Basic___hyg_62____closed__41; LEAN_EXPORT lean_object* l_Lean_Language_withHeaderExceptions(lean_object*); @@ -246,6 +249,7 @@ uint8_t lean_nat_dec_lt(lean_object*, lean_object*); static lean_object* l___auto____x40_Lean_Language_Basic___hyg_62____closed__27; LEAN_EXPORT lean_object* l_Lean_Language_withAlwaysResolvedPromises___rarg___lambda__1___boxed(lean_object*, lean_object*); static lean_object* l___auto____x40_Lean_Language_Basic___hyg_62____closed__25; +static lean_object* l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__1; LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Language_SnapshotTree_trace_go___spec__5___lambda__2(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, double, double, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_forMAux___at_Lean_Language_reportMessages___spec__3___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); @@ -275,6 +279,7 @@ lean_object* l_List_reverse___rarg(lean_object*); static lean_object* l_Lean_Language_withAlwaysResolvedPromise___rarg___closed__1; lean_object* lean_array_mk(lean_object*); static lean_object* l_Lean_Language_SnapshotTree_trace_go___closed__8; +LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Language_withAlwaysResolvedPromises___spec__2___rarg___lambda__1(lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); static lean_object* l___auto____x40_Lean_Language_Basic___hyg_62____closed__18; @@ -287,8 +292,8 @@ extern lean_object* l_Lean_trace_profiler; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Language_withAlwaysResolvedPromises___spec__1___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_SnapshotTask_get___rarg(lean_object*); lean_object* l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_compileDecl___spec__4___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_SnapshotTree_trace(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__4; LEAN_EXPORT lean_object* l_Lean_Language_mkIncrementalProcessor___elambda__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_io_error_to_string(lean_object*); lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); @@ -313,6 +318,7 @@ static lean_object* l___auto____x40_Lean_Language_Basic___hyg_62____closed__32; LEAN_EXPORT lean_object* l_Std_Format_prefixJoin___at_Lean_Language_SnapshotTree_trace_go___spec__2(lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_SnapshotTask_bindIO___rarg___lambda__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Language_instInhabitedDynamicSnapshot___spec__1___lambda__1(lean_object*, lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); static lean_object* l___auto____x40_Lean_Language_Basic___hyg_62____closed__6; LEAN_EXPORT lean_object* l_Lean_Language_SnapshotTask_cancel(lean_object*); @@ -4984,10 +4990,10 @@ return x_3; LEAN_EXPORT lean_object* l_Lean_Language_instToSnapshotTreeDynamicSnapshot(lean_object* x_1) { _start: { -lean_object* x_2; +lean_object* x_2; lean_object* x_3; x_2 = lean_ctor_get(x_1, 1); -lean_inc(x_2); -return x_2; +x_3 = lean_thunk_get_own(x_2); +return x_3; } } LEAN_EXPORT lean_object* l_Lean_Language_instToSnapshotTreeDynamicSnapshot___boxed(lean_object* x_1) { @@ -4999,19 +5005,30 @@ lean_dec(x_1); return x_2; } } +LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = lean_apply_1(x_1, x_2); +return x_4; +} +} LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_4; lean_object* x_5; lean_object* x_6; +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_inc(x_3); x_4 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_3); -x_5 = lean_apply_1(x_2, x_3); -x_6 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_6, 0, x_4); -lean_ctor_set(x_6, 1, x_5); -return x_6; +x_5 = lean_alloc_closure((void*)(l_Lean_Language_DynamicSnapshot_ofTyped___rarg___lambda__1___boxed), 3, 2); +lean_closure_set(x_5, 0, x_2); +lean_closure_set(x_5, 1, x_3); +x_6 = lean_mk_thunk(x_5); +x_7 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_7, 0, x_4); +lean_ctor_set(x_7, 1, x_6); +return x_7; } } LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped(lean_object* x_1) { @@ -5022,6 +5039,15 @@ x_2 = lean_alloc_closure((void*)(l_Lean_Language_DynamicSnapshot_ofTyped___rarg) return x_2; } } +LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Lean_Language_DynamicSnapshot_ofTyped___rarg___lambda__1(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; +} +} LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_toTyped_x3f___rarg(lean_object* x_1, lean_object* x_2) { _start: { @@ -5049,6 +5075,17 @@ lean_dec(x_1); return x_3; } } +LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Language_instInhabitedDynamicSnapshot___spec__1___lambda__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; +x_3 = l_Lean_addTrace___at_Lean_Language_SnapshotTree_trace_go___spec__7___closed__1; +x_4 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_3); +return x_4; +} +} LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Language_instInhabitedDynamicSnapshot___spec__1(lean_object* x_1, lean_object* x_2) { _start: { @@ -5057,10 +5094,9 @@ lean_inc(x_2); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); -x_4 = l_Lean_addTrace___at_Lean_Language_SnapshotTree_trace_go___spec__7___closed__1; -x_5 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_5, 0, x_2); -lean_ctor_set(x_5, 1, x_4); +x_4 = lean_alloc_closure((void*)(l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Language_instInhabitedDynamicSnapshot___spec__1___lambda__1___boxed), 2, 1); +lean_closure_set(x_4, 0, x_2); +x_5 = lean_mk_thunk(x_4); x_6 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_6, 0, x_3); lean_ctor_set(x_6, 1, x_5); @@ -5139,6 +5175,15 @@ x_3 = l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Language_instInhabitedDy return x_3; } } +LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Language_instInhabitedDynamicSnapshot___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Language_instInhabitedDynamicSnapshot___spec__1___lambda__1(x_1, x_2); +lean_dec(x_2); +return x_3; +} +} LEAN_EXPORT lean_object* l_Lean_Language_instInhabitedDynamicSnapshot___lambda__1___boxed(lean_object* x_1) { _start: { @@ -5265,7 +5310,7 @@ lean_dec(x_4); return x_5; } } -static lean_object* _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__1() { +static lean_object* _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__1() { _start: { lean_object* x_1; @@ -5273,17 +5318,17 @@ x_1 = lean_mk_string_unchecked("printMessageEndPos", 18, 18); return x_1; } } -static lean_object* _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__2() { +static lean_object* _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__1; +x_2 = l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__3() { +static lean_object* _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__3() { _start: { lean_object* x_1; @@ -5291,13 +5336,13 @@ x_1 = lean_mk_string_unchecked("print end position of each message in addition t return x_1; } } -static lean_object* _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__4() { +static lean_object* _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__4() { _start: { uint8_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = 0; x_2 = l_Lean_Language_instInhabitedSnapshot___closed__1; -x_3 = l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__3; +x_3 = l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__3; x_4 = lean_box(x_1); x_5 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_5, 0, x_4); @@ -5306,24 +5351,24 @@ lean_ctor_set(x_5, 2, x_3); return x_5; } } -static lean_object* _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__5() { +static lean_object* _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l___auto____x40_Lean_Language_Basic___hyg_62____closed__1; x_2 = l_Lean_Language_instImpl____x40_Lean_Language_Basic___hyg_1850____closed__1; -x_3 = l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__1; +x_3 = l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__1; x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_2 = l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__2; -x_3 = l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__4; -x_4 = l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__5; +x_2 = l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__2; +x_3 = l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__4; +x_4 = l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__5; x_5 = l_Lean_Option_register___at_Lean_initFn____x40_Lean_Util_Profile___hyg_5____spec__1(x_2, x_3, x_4, x_1); return x_5; } @@ -7162,17 +7207,17 @@ l_Lean_Language_instInhabitedDynamicSnapshot___closed__5 = _init_l_Lean_Language lean_mark_persistent(l_Lean_Language_instInhabitedDynamicSnapshot___closed__5); l_Lean_Language_instInhabitedDynamicSnapshot = _init_l_Lean_Language_instInhabitedDynamicSnapshot(); lean_mark_persistent(l_Lean_Language_instInhabitedDynamicSnapshot); -l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__1 = _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__1(); -lean_mark_persistent(l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__1); -l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__2 = _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__2(); -lean_mark_persistent(l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__2); -l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__3 = _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__3(); -lean_mark_persistent(l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__3); -l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__4 = _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__4(); -lean_mark_persistent(l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__4); -l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__5 = _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__5(); -lean_mark_persistent(l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__5); -if (builtin) {res = l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057_(lean_io_mk_world()); +l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__1 = _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__1(); +lean_mark_persistent(l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__1); +l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__2 = _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__2(); +lean_mark_persistent(l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__2); +l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__3 = _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__3(); +lean_mark_persistent(l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__3); +l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__4 = _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__4(); +lean_mark_persistent(l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__4); +l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__5 = _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__5(); +lean_mark_persistent(l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__5); +if (builtin) {res = l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_Language_printMessageEndPos = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Language_printMessageEndPos); diff --git a/stage0/stdlib/Lean/Language/Lean.c b/stage0/stdlib/Lean/Language/Lean.c index 5fe08cccd806..5c795550af76 100644 --- a/stage0/stdlib/Lean/Language/Lean.c +++ b/stage0/stdlib/Lean/Language/Lean.c @@ -13,24 +13,26 @@ #ifdef __cplusplus extern "C" { #endif -static size_t l_Lean_Language_Lean_process_processHeader___lambda__5___closed__3; -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_processHeader___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_processHeader___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_Lean_process(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_Lean_initFn____x40_Lean_Language_Lean___hyg_437_(lean_object*); lean_object* lean_profileit(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Language_Lean_reparseOptions___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Language_Lean_reparseOptions___spec__1___lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_processHeader___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_Language_Lean_initFn____x40_Lean_Language_Lean___hyg_10____closed__6; -lean_object* l_EIO_toBaseIO___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_processHeader___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, double, double, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_processHeader___lambda__5(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_Language_Lean_initFn____x40_Lean_Language_Lean___hyg_10____closed__2; static lean_object* l_Lean_Language_Lean_process_parseHeader___lambda__3___closed__3; static lean_object* l_Lean_Language_Lean_process_doElab___lambda__3___closed__1; -static lean_object* l_Lean_Language_Lean_process_processHeader___lambda__5___closed__2; +static lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__4___closed__1; +static lean_object* l_Lean_Language_Lean_process_processHeader___lambda__3___closed__10; static lean_object* l_IO_FS_withIsolatedStreams___at_Lean_Language_Lean_process_doElab___spec__1___closed__4; +static lean_object* l_Lean_Language_Lean_process_processHeader___lambda__3___closed__8; lean_object* l_Lean_Language_Snapshot_Diagnostics_ofMessageLog(lean_object*, lean_object*); double lean_float_div(double, double); +static lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__5___closed__2; lean_object* lean_io_promise_new(lean_object*); lean_object* l_String_toNat_x3f(lean_object*); lean_object* lean_get_set_stdout(lean_object*, lean_object*); @@ -39,37 +41,44 @@ lean_object* l_Lean_FileMap_toPosition(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_Language_Lean_process_processHeader___spec__2(lean_object*, lean_object*); lean_object* l_Lean_Elab_Command_elabCommandTopLevel(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_io_as_task(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Language_Lean_process_processHeader___lambda__3___closed__5; static lean_object* l_Lean_Language_Lean_initFn____x40_Lean_Language_Lean___hyg_437____closed__5; lean_object* l_Lean_Name_toString(lean_object*, uint8_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Language_Lean_process_processHeader___lambda__3___closed__7; +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__7(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Language_Lean_process_processHeader___lambda__4___closed__2; static lean_object* l___private_Lean_Language_Lean_0__Lean_Language_Lean_withHeaderExceptions___rarg___closed__13; LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseHeader___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__7___closed__1; LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_processHeader(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Language_Lean_process_processHeader___lambda__5___closed__7; +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__2___closed__2; lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Language_instInhabitedDynamicSnapshot___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseHeader___lambda__1(lean_object*, lean_object*); static lean_object* l_List_mapTR_loop___at_Lean_Language_Lean_process_processHeader___spec__1___closed__3; lean_object* l_Lean_Elab_Command_mkState(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_Lean_LeanProcessingM_run(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_processHeader___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_processHeader___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getArgs(lean_object*); static lean_object* l_Lean_Language_Lean_process_parseHeader___lambda__3___closed__1; lean_object* l_Lean_Language_SnapshotTask_ofIO___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Language_Lean_0__Lean_Language_Lean_withHeaderExceptions___rarg___closed__7; -static lean_object* l_Lean_Language_Lean_process_parseCmd___closed__1; +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__9___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_Lean_Language_Lean_reparseOptions___spec__1___lambda__1___closed__3; static lean_object* l_Lean_Language_Lean_process_processHeader___lambda__4___closed__10; lean_object* l_Lean_Syntax_getTailPos_x3f(lean_object*, uint8_t); +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Language_Lean_process_processHeader___lambda__3___closed__3; static lean_object* l_IO_FS_withIsolatedStreams___at_Lean_Language_Lean_process_doElab___spec__1___closed__1; +static lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__5___closed__3; static lean_object* l_List_forIn_loop___at_Lean_Language_Lean_reparseOptions___spec__1___lambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Language_Lean_0__Lean_Language_Lean_withHeaderExceptions___rarg___closed__6; -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Language_Lean_process_processHeader___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_Lean_reparseOptions(lean_object*, lean_object*); +static lean_object* l_Lean_Language_Lean_process_processHeader___lambda__3___closed__1; +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Language_Lean_0__Lean_Language_Lean_withHeaderExceptions___rarg___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseHeader___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_doElab(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -77,17 +86,18 @@ lean_object* l_Lean_Name_mkStr5(lean_object*, lean_object*, lean_object*, lean_o size_t lean_usize_of_nat(lean_object*); lean_object* l_Lean_Elab_processHeader(lean_object*, lean_object*, lean_object*, lean_object*, uint32_t, uint8_t, lean_object*); lean_object* lean_io_promise_result(lean_object*); +static lean_object* l_Lean_Language_Lean_process_processHeader___lambda__3___closed__2; extern lean_object* l_Lean_maxRecDepth; lean_object* l_Lean_KVMap_insertCore(lean_object*, lean_object*, lean_object*); lean_object* l_List_head_x21___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Language_Lean_process_doElab___lambda__4___closed__2; uint8_t lean_string_dec_eq(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__8(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Language_Lean_reparseOptions___spec__1___lambda__1___closed__5; static lean_object* l_List_forIn_loop___at_Lean_Language_Lean_reparseOptions___spec__1___closed__1; static lean_object* l_Lean_Language_Lean_process_doElab___lambda__3___closed__2; lean_object* lean_string_utf8_byte_size(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_string_validate_utf8(lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseHeader(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseHeader___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -100,6 +110,7 @@ lean_object* l_Lean_Elab_withLogging___at_Lean_Elab_Command_elabCommand___spec__ static lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__2___closed__4; LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseHeader___lambda__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_io_promise_resolve(lean_object*, lean_object*, lean_object*); +lean_object* l_IO_Promise_new___boxed(lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Elab_instInhabitedInfoTree; uint8_t l_Lean_Parser_isTerminalCommand(lean_object*); lean_object* l_IO_CancelToken_new(lean_object*); @@ -111,14 +122,13 @@ lean_object* lean_st_ref_take(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_Lean_processCommands(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Language_Lean_0__Lean_Language_Lean_withHeaderExceptions___rarg___closed__5; LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseHeader___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Language_Lean_process_doElab___lambda__4___closed__6; extern lean_object* l_ByteArray_empty; -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_processHeader___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_processHeader___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_List_toPArray_x27___rarg(lean_object*); lean_object* l_Lean_Option_get___at_Lean_profiler_threshold_getSecs___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Language_Lean_initFn____x40_Lean_Language_Lean___hyg_437____closed__6; -static double l_Lean_Language_Lean_process_processHeader___lambda__6___closed__1; LEAN_EXPORT lean_object* l_Lean_Language_Lean_instMonadLiftLeanProcessingMLeanProcessingTIO(lean_object*); static lean_object* l_Lean_Language_Lean_process_doElab___closed__3; static lean_object* l_List_mapTR_loop___at_Lean_Language_Lean_process_processHeader___spec__1___closed__2; @@ -138,7 +148,6 @@ LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_doElab___boxed(lean_object lean_object* l_Lean_Name_replacePrefix(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Language_Lean_reparseOptions___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); -static lean_object* l_Lean_Language_Lean_process_processHeader___lambda__5___closed__10; LEAN_EXPORT lean_object* l_Lean_Language_Lean_initFn____x40_Lean_Language_Lean___hyg_10_(lean_object*); static lean_object* l_Lean_Language_Lean_process_processHeader___lambda__4___closed__9; LEAN_EXPORT lean_object* l_Lean_Language_Lean_LeanProcessingM_run___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -149,7 +158,7 @@ lean_object* lean_array_to_list(lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Language_Lean_reparseOptions___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_Name_num___override(lean_object*, lean_object*); lean_object* l_Lean_Name_append(lean_object*, lean_object*); -static lean_object* l_Lean_Language_Lean_process_processHeader___lambda__5___closed__1; +static double l_Lean_Language_Lean_process_processHeader___lambda__5___closed__1; static lean_object* l_List_forIn_loop___at_Lean_Language_Lean_reparseOptions___spec__1___lambda__1___closed__4; static lean_object* l___private_Lean_Language_Lean_0__Lean_Language_Lean_withHeaderExceptions___rarg___closed__4; LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_processHeader___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -165,11 +174,13 @@ lean_object* l_Lean_Language_diagnosticsOfHeaderError(lean_object*, lean_object* extern lean_object* l_Task_Priority_default; static lean_object* l_List_forIn_loop___at_Lean_Language_Lean_reparseOptions___spec__1___lambda__1___closed__7; LEAN_EXPORT lean_object* l___private_Lean_Language_Lean_0__Lean_Language_Lean_withHeaderExceptions___rarg___lambda__1___boxed(lean_object*); +static lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__9___closed__1; uint8_t lean_name_eq(lean_object*, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_doElab___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* l_IO_FS_Stream_ofBuffer(lean_object*); static lean_object* l___private_Lean_Language_Lean_0__Lean_Language_Lean_withHeaderExceptions___rarg___closed__12; +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__9(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_Lean_waitForFinalCmdState_x3f_goCmd(lean_object*); extern lean_object* l_Lean_MessageLog_empty; uint8_t l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(lean_object*, lean_object*); @@ -178,18 +189,18 @@ static lean_object* l_Lean_Language_Lean_initFn____x40_Lean_Language_Lean___hyg_ lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Language_Lean_process_doElab___lambda__3___closed__7; -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__4(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_get_set_stderr(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_Lean_internal_cmdlineSnapshots; static lean_object* l_Lean_Language_Lean_process_processHeader___closed__1; extern lean_object* l_Lean_Language_Snapshot_Diagnostics_empty; -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseHeader___lambda__2(lean_object*, lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Language_Lean_reparseOptions___spec__1___lambda__1___closed__10; static lean_object* l_Lean_Language_Lean_initFn____x40_Lean_Language_Lean___hyg_437____closed__2; lean_object* lean_string_from_utf8_unchecked(lean_object*); -static lean_object* l_Lean_Language_Lean_process_processHeader___lambda__4___closed__3; -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_processHeader___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 size_t l_Lean_Language_Lean_process_processHeader___lambda__4___closed__3; +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_processHeader___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, double, double, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Language_Lean_0__Lean_Language_Lean_withHeaderExceptions___rarg___closed__3; static lean_object* l_Lean_Language_Lean_process_processHeader___lambda__4___closed__4; static lean_object* l___private_Lean_Language_Lean_0__Lean_Language_Lean_withHeaderExceptions___rarg___closed__9; @@ -197,24 +208,24 @@ lean_object* l_Lean_Option_register___at_Lean_Elab_initFn____x40_Lean_Elab_AutoB LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_doElab___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_doElab___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*); double l_Float_ofScientific(lean_object*, uint8_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___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_Language_Lean_process_parseCmd___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_doElab___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_processHeader___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_KVMap_erase(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Language_Lean_reparseOptions___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Language_Lean_process_doElab___closed__1; extern lean_object* l_Lean_NameSet_empty; LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseHeader___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Language_Lean_0__Lean_Language_Lean_withHeaderExceptions___rarg___closed__10; static lean_object* l_Lean_Language_Lean_process_processHeader___lambda__4___closed__1; -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_processHeader___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); static lean_object* l_Lean_Language_Lean_process_doElab___lambda__3___closed__8; uint8_t lean_nat_dec_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_Lean_instMonadLiftLeanProcessingMLeanProcessingTIO___rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_Lean_isBeforeEditPos(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Language_Lean_process_processHeader___lambda__3___closed__4; lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseHeader___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_IO_FS_withIsolatedStreams___at_Lean_Language_Lean_process_doElab___spec__1(lean_object*, uint8_t, lean_object*, lean_object*); @@ -222,40 +233,37 @@ static lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__5___closed__ static lean_object* l___private_Lean_Language_Lean_0__Lean_Language_Lean_withHeaderExceptions___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseHeader___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_Lean_stderrAsMessages; -static lean_object* l_Lean_Language_Lean_process_processHeader___lambda__5___closed__5; lean_object* l_Lean_Language_SnapshotTask_get_x3f___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_processHeader___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_Lean_waitForFinalCmdState_x3f(lean_object*); static lean_object* l_Lean_Language_Lean_initFn____x40_Lean_Language_Lean___hyg_437____closed__7; -static lean_object* l_Lean_Language_Lean_process_processHeader___lambda__5___closed__9; lean_object* l_Lean_Language_SnapshotTask_bindIO___rarg(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*); static lean_object* l_Lean_Language_Lean_process_parseHeader___lambda__3___closed__2; static lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__2___closed__1; -static lean_object* l_Lean_Language_Lean_process_parseCmd___closed__3; static lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__2___closed__3; LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Language_Lean_process_doElab___closed__2; static lean_object* l_List_forIn_loop___at_Lean_Language_Lean_reparseOptions___spec__1___lambda__1___closed__2; static lean_object* l_List_forIn_loop___at_Lean_Language_Lean_reparseOptions___spec__1___closed__2; static lean_object* l___private_Lean_Language_Lean_0__Lean_Language_Lean_withHeaderExceptions___rarg___closed__11; -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___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_get_set_stdin(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_Language_Lean_process_processHeader___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getRange_x3f(lean_object*, uint8_t); lean_object* l_Lean_Option_get_x3f___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessages___spec__1(lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Language_Lean_reparseOptions___spec__1___lambda__1___closed__11; LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseHeader___lambda__2___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__5(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Language_Lean_process_doElab___lambda__3___closed__5; +static lean_object* l_Lean_Language_Lean_process_processHeader___lambda__3___closed__9; LEAN_EXPORT lean_object* l_Lean_Language_Lean_isBeforeEditPos___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); -static lean_object* l_Lean_Language_Lean_process_parseCmd___closed__2; static lean_object* l_Lean_Language_Lean_initFn____x40_Lean_Language_Lean___hyg_10____closed__5; static lean_object* l_Lean_Language_Lean_initFn____x40_Lean_Language_Lean___hyg_10____closed__4; +static lean_object* l_Lean_Language_Lean_process_processHeader___lambda__3___closed__6; static lean_object* l_Lean_Language_Lean_initFn____x40_Lean_Language_Lean___hyg_10____closed__1; lean_object* l_List_reverse___rarg(lean_object*); static lean_object* l_Lean_Language_Lean_process_doElab___lambda__3___closed__6; -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_firstFrontendMacroScope; static lean_object* l_IO_FS_withIsolatedStreams___at_Lean_Language_Lean_process_doElab___spec__1___closed__2; extern lean_object* l_Lean_Elab_Command_instInhabitedScope; @@ -265,9 +273,7 @@ lean_object* l_Lean_PersistentArray_get_x21___rarg(lean_object*, lean_object*, l LEAN_EXPORT lean_object* l_IO_withStderr___at_Lean_Language_Lean_process_doElab___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_eqWithInfo(lean_object*, lean_object*); static lean_object* l_IO_FS_withIsolatedStreams___at_Lean_Language_Lean_process_doElab___spec__1___closed__5; -static lean_object* l_Lean_Language_Lean_process_processHeader___lambda__5___closed__4; static lean_object* l_Lean_Language_Lean_process_doElab___lambda__4___closed__5; -static lean_object* l_Lean_Language_Lean_process_processHeader___lambda__5___closed__6; static lean_object* l_Lean_Language_Lean_initFn____x40_Lean_Language_Lean___hyg_437____closed__3; lean_object* l_Lean_Language_SnapshotTask_get___rarg(lean_object*); lean_object* lean_io_error_to_string(lean_object*); @@ -284,13 +290,13 @@ lean_object* l_Lean_RBNode_find___at_Lean_NameMap_find_x3f___spec__1___rarg(lean static lean_object* l_List_forIn_loop___at_Lean_Language_Lean_reparseOptions___spec__1___lambda__1___closed__8; lean_object* lean_nat_add(lean_object*, lean_object*); lean_object* lean_runtime_mark_persistent(lean_object*); +lean_object* l_EStateM_bind___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Language_Lean_process_processHeader___lambda__4___closed__7; static lean_object* l_List_forIn_loop___at_Lean_Language_Lean_reparseOptions___spec__1___lambda__1___closed__9; lean_object* l_Lean_Parser_parseCommand(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseHeader___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Language_Lean_process_doElab___lambda__4___closed__1; LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_processHeader___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Language_Lean_process_processHeader___lambda__5___closed__8; LEAN_EXPORT lean_object* l___private_Lean_Language_Lean_0__Lean_Language_Lean_withHeaderExceptions(lean_object*); static lean_object* l_Lean_Language_Lean_process_doElab___lambda__4___closed__4; static lean_object* l___private_Lean_Language_Lean_0__Lean_Language_Lean_withHeaderExceptions___rarg___closed__8; @@ -4574,217 +4580,218 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___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, uint8_t x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___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, uint8_t x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { -lean_object* x_17; -x_17 = l_Lean_Language_Snapshot_Diagnostics_ofMessageLog(x_1, x_16); -if (lean_obj_tag(x_17) == 0) +lean_object* x_16; +x_16 = l_Lean_Language_Snapshot_Diagnostics_ofMessageLog(x_1, x_15); +if (lean_obj_tag(x_16) == 0) { -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_17, 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); -x_19 = lean_ctor_get(x_17, 1); -lean_inc(x_19); -lean_dec(x_17); +lean_dec(x_16); if (x_12 == 0) { -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; -x_126 = lean_box(0); -x_127 = l_Lean_Language_Lean_process_parseCmd___lambda__2___closed__3; -x_128 = 0; -x_129 = lean_alloc_ctor(0, 3, 1); -lean_ctor_set(x_129, 0, x_127); -lean_ctor_set(x_129, 1, x_18); -lean_ctor_set(x_129, 2, x_126); -lean_ctor_set_uint8(x_129, sizeof(void*)*3, x_128); -x_130 = l_Lean_Syntax_getRange_x3f(x_5, x_128); -lean_inc(x_4); -x_131 = lean_io_promise_result(x_4); -x_132 = lean_alloc_ctor(0, 2, 0); +lean_object* x_129; lean_object* x_130; uint8_t x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; +x_129 = lean_box(0); +x_130 = l_Lean_Language_Lean_process_parseCmd___lambda__2___closed__3; +x_131 = 0; +x_132 = lean_alloc_ctor(0, 3, 1); lean_ctor_set(x_132, 0, x_130); -lean_ctor_set(x_132, 1, x_131); +lean_ctor_set(x_132, 1, x_17); +lean_ctor_set(x_132, 2, x_129); +lean_ctor_set_uint8(x_132, sizeof(void*)*3, x_131); +x_133 = l_Lean_Syntax_getRange_x3f(x_5, x_131); +lean_inc(x_4); +x_134 = lean_io_promise_result(x_4); +x_135 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_135, 0, x_133); +lean_ctor_set(x_135, 1, x_134); lean_inc(x_9); lean_inc(x_11); lean_inc(x_5); -x_133 = lean_alloc_ctor(0, 6, 0); -lean_ctor_set(x_133, 0, x_129); -lean_ctor_set(x_133, 1, x_5); -lean_ctor_set(x_133, 2, x_11); -lean_ctor_set(x_133, 3, x_132); -lean_ctor_set(x_133, 4, x_13); -lean_ctor_set(x_133, 5, x_9); -x_20 = x_133; -goto block_125; +x_136 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_136, 0, x_132); +lean_ctor_set(x_136, 1, x_5); +lean_ctor_set(x_136, 2, x_11); +lean_ctor_set(x_136, 3, x_135); +lean_ctor_set(x_136, 4, x_13); +lean_ctor_set(x_136, 5, x_9); +x_19 = x_136; +goto block_128; } else { -uint8_t x_134; +uint8_t x_137; lean_inc(x_5); -x_134 = l_Lean_Parser_isTerminalCommand(x_5); -if (x_134 == 0) -{ -lean_object* x_135; lean_object* x_136; uint8_t x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; -x_135 = lean_box(0); -x_136 = l_Lean_Language_Lean_process_parseCmd___lambda__2___closed__3; -x_137 = 0; -x_138 = lean_alloc_ctor(0, 3, 1); -lean_ctor_set(x_138, 0, x_136); -lean_ctor_set(x_138, 1, x_18); -lean_ctor_set(x_138, 2, x_135); -lean_ctor_set_uint8(x_138, sizeof(void*)*3, x_137); -x_139 = l_Lean_Syntax_getRange_x3f(x_5, x_137); -lean_inc(x_4); -x_140 = lean_io_promise_result(x_4); -x_141 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_141, 0, x_139); -lean_ctor_set(x_141, 1, x_140); -x_142 = lean_box(0); -x_143 = l_Lean_Language_Lean_process_parseCmd___lambda__2___closed__4; -lean_inc(x_9); -x_144 = lean_alloc_ctor(0, 6, 0); -lean_ctor_set(x_144, 0, x_138); -lean_ctor_set(x_144, 1, x_142); -lean_ctor_set(x_144, 2, x_143); -lean_ctor_set(x_144, 3, x_141); -lean_ctor_set(x_144, 4, x_13); -lean_ctor_set(x_144, 5, x_9); -x_20 = x_144; -goto block_125; -} -else +x_137 = l_Lean_Parser_isTerminalCommand(x_5); +if (x_137 == 0) { -lean_object* x_145; lean_object* x_146; uint8_t x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; -x_145 = lean_box(0); -x_146 = l_Lean_Language_Lean_process_parseCmd___lambda__2___closed__3; -x_147 = 0; -x_148 = lean_alloc_ctor(0, 3, 1); -lean_ctor_set(x_148, 0, x_146); -lean_ctor_set(x_148, 1, x_18); -lean_ctor_set(x_148, 2, x_145); -lean_ctor_set_uint8(x_148, sizeof(void*)*3, x_147); -x_149 = l_Lean_Syntax_getRange_x3f(x_5, x_147); +lean_object* x_138; lean_object* x_139; uint8_t x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; +x_138 = lean_box(0); +x_139 = l_Lean_Language_Lean_process_parseCmd___lambda__2___closed__3; +x_140 = 0; +x_141 = lean_alloc_ctor(0, 3, 1); +lean_ctor_set(x_141, 0, x_139); +lean_ctor_set(x_141, 1, x_17); +lean_ctor_set(x_141, 2, x_138); +lean_ctor_set_uint8(x_141, sizeof(void*)*3, x_140); +x_142 = l_Lean_Syntax_getRange_x3f(x_5, x_140); lean_inc(x_4); -x_150 = lean_io_promise_result(x_4); -x_151 = lean_alloc_ctor(0, 2, 0); +x_143 = lean_io_promise_result(x_4); +x_144 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_144, 0, x_142); +lean_ctor_set(x_144, 1, x_143); +x_145 = lean_box(0); +x_146 = l_Lean_Language_Lean_process_parseCmd___lambda__2___closed__4; +lean_inc(x_9); +x_147 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_147, 0, x_141); +lean_ctor_set(x_147, 1, x_145); +lean_ctor_set(x_147, 2, x_146); +lean_ctor_set(x_147, 3, x_144); +lean_ctor_set(x_147, 4, x_13); +lean_ctor_set(x_147, 5, x_9); +x_19 = x_147; +goto block_128; +} +else +{ +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; lean_object* x_155; +x_148 = lean_box(0); +x_149 = l_Lean_Language_Lean_process_parseCmd___lambda__2___closed__3; +x_150 = 0; +x_151 = lean_alloc_ctor(0, 3, 1); lean_ctor_set(x_151, 0, x_149); -lean_ctor_set(x_151, 1, x_150); +lean_ctor_set(x_151, 1, x_17); +lean_ctor_set(x_151, 2, x_148); +lean_ctor_set_uint8(x_151, sizeof(void*)*3, x_150); +x_152 = l_Lean_Syntax_getRange_x3f(x_5, x_150); +lean_inc(x_4); +x_153 = lean_io_promise_result(x_4); +x_154 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_154, 0, x_152); +lean_ctor_set(x_154, 1, x_153); lean_inc(x_9); lean_inc(x_11); lean_inc(x_5); -x_152 = lean_alloc_ctor(0, 6, 0); -lean_ctor_set(x_152, 0, x_148); -lean_ctor_set(x_152, 1, x_5); -lean_ctor_set(x_152, 2, x_11); -lean_ctor_set(x_152, 3, x_151); -lean_ctor_set(x_152, 4, x_13); -lean_ctor_set(x_152, 5, x_9); -x_20 = x_152; -goto block_125; +x_155 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_155, 0, x_151); +lean_ctor_set(x_155, 1, x_5); +lean_ctor_set(x_155, 2, x_11); +lean_ctor_set(x_155, 3, x_154); +lean_ctor_set(x_155, 4, x_13); +lean_ctor_set(x_155, 5, x_9); +x_19 = x_155; +goto block_128; } } -block_125: +block_128: { -lean_object* x_21; +lean_object* x_20; if (lean_obj_tag(x_14) == 0) { -lean_object* x_114; -x_114 = lean_box(0); -x_21 = x_114; -goto block_113; +lean_object* x_117; +x_117 = lean_box(0); +x_20 = x_117; +goto block_116; } 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; -x_115 = lean_ctor_get(x_14, 0); -lean_inc(x_115); -x_116 = lean_ctor_get(x_11, 0); -lean_inc(x_116); -x_117 = lean_ctor_get(x_10, 0); -lean_inc(x_117); -x_118 = lean_ctor_get(x_117, 0); +lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; +x_118 = lean_ctor_get(x_14, 0); lean_inc(x_118); -lean_dec(x_117); -x_119 = lean_string_utf8_byte_size(x_118); -lean_dec(x_118); -x_120 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_120, 0, x_116); -lean_ctor_set(x_120, 1, x_119); -x_121 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_121, 0, x_120); -x_122 = lean_io_promise_result(x_115); +x_119 = lean_ctor_get(x_11, 0); +lean_inc(x_119); +x_120 = lean_ctor_get(x_10, 0); +lean_inc(x_120); +x_121 = lean_ctor_get(x_120, 0); +lean_inc(x_121); +lean_dec(x_120); +x_122 = lean_string_utf8_byte_size(x_121); +lean_dec(x_121); x_123 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_123, 0, x_121); +lean_ctor_set(x_123, 0, x_119); lean_ctor_set(x_123, 1, x_122); x_124 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_124, 0, x_123); -x_21 = x_124; -goto block_113; +x_125 = lean_io_promise_result(x_118); +x_126 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_126, 0, x_124); +lean_ctor_set(x_126, 1, x_125); +x_127 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_127, 0, x_126); +x_20 = x_127; +goto block_116; } -block_113: +block_116: { -lean_object* x_22; lean_object* x_23; -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_io_promise_resolve(x_22, x_2, x_19); -if (lean_obj_tag(x_23) == 0) +lean_object* x_21; lean_object* x_22; +x_21 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_21, 0, x_19); +lean_ctor_set(x_21, 1, x_20); +x_22 = lean_io_promise_resolve(x_21, x_2, x_18); +if (lean_obj_tag(x_22) == 0) { if (lean_obj_tag(x_3) == 0) { -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_24 = lean_ctor_get(x_23, 1); -lean_inc(x_24); -lean_dec(x_23); -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_4); +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_23 = lean_ctor_get(x_22, 1); +lean_inc(x_23); +lean_dec(x_22); +x_24 = lean_box(0); +x_25 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_25, 0, x_24); +lean_ctor_set(x_25, 1, x_4); lean_inc(x_10); -x_27 = l_Lean_Language_Lean_process_doElab(x_5, x_6, x_7, x_26, x_8, x_9, x_10, x_24); +x_26 = l_Lean_Language_Lean_process_doElab(x_5, x_6, x_7, x_25, x_8, x_9, x_10, x_23); lean_dec(x_9); -if (lean_obj_tag(x_27) == 0) +if (lean_obj_tag(x_26) == 0) { if (lean_obj_tag(x_14) == 0) { -uint8_t x_28; +uint8_t x_27; lean_dec(x_11); lean_dec(x_10); -x_28 = !lean_is_exclusive(x_27); -if (x_28 == 0) +x_27 = !lean_is_exclusive(x_26); +if (x_27 == 0) { -lean_object* x_29; lean_object* x_30; -x_29 = lean_ctor_get(x_27, 0); -lean_dec(x_29); -x_30 = lean_box(0); -lean_ctor_set(x_27, 0, x_30); -return x_27; +lean_object* x_28; lean_object* x_29; +x_28 = lean_ctor_get(x_26, 0); +lean_dec(x_28); +x_29 = lean_box(0); +lean_ctor_set(x_26, 0, x_29); +return x_26; } else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_31 = lean_ctor_get(x_27, 1); -lean_inc(x_31); -lean_dec(x_27); -x_32 = lean_box(0); -x_33 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_33, 0, x_32); -lean_ctor_set(x_33, 1, x_31); -return x_33; +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_26, 1); +lean_inc(x_30); +lean_dec(x_26); +x_31 = lean_box(0); +x_32 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_32, 0, x_31); +lean_ctor_set(x_32, 1, x_30); +return x_32; } } else { -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_34 = lean_ctor_get(x_27, 0); +lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; lean_object* x_37; +x_33 = lean_ctor_get(x_26, 0); +lean_inc(x_33); +x_34 = lean_ctor_get(x_26, 1); lean_inc(x_34); -x_35 = lean_ctor_get(x_27, 1); +lean_dec(x_26); +x_35 = lean_ctor_get(x_14, 0); lean_inc(x_35); -lean_dec(x_27); -x_36 = lean_ctor_get(x_14, 0); -lean_inc(x_36); lean_dec(x_14); -x_37 = l_Lean_Language_Lean_process_parseCmd(x_25, x_11, x_34, x_36, x_10, x_35); +x_36 = 0; +x_37 = l_Lean_Language_Lean_process_parseCmd(x_24, x_11, x_33, x_35, x_36, x_10, x_34); return x_37; } } @@ -4794,19 +4801,19 @@ uint8_t x_38; lean_dec(x_14); lean_dec(x_11); lean_dec(x_10); -x_38 = !lean_is_exclusive(x_27); +x_38 = !lean_is_exclusive(x_26); if (x_38 == 0) { -return x_27; +return x_26; } else { lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_39 = lean_ctor_get(x_27, 0); -x_40 = lean_ctor_get(x_27, 1); +x_39 = lean_ctor_get(x_26, 0); +x_40 = lean_ctor_get(x_26, 1); lean_inc(x_40); lean_inc(x_39); -lean_dec(x_27); +lean_dec(x_26); x_41 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_41, 0, x_39); lean_ctor_set(x_41, 1, x_40); @@ -4822,9 +4829,9 @@ if (x_42 == 0) { lean_object* x_43; lean_object* x_44; uint8_t x_45; x_43 = lean_ctor_get(x_3, 0); -x_44 = lean_ctor_get(x_23, 1); +x_44 = lean_ctor_get(x_22, 1); lean_inc(x_44); -lean_dec(x_23); +lean_dec(x_22); x_45 = !lean_is_exclusive(x_43); if (x_45 == 0) { @@ -4877,7 +4884,7 @@ return x_57; } else { -lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; +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_ctor_get(x_51, 0); lean_inc(x_58); x_59 = lean_ctor_get(x_51, 1); @@ -4887,244 +4894,247 @@ x_60 = lean_ctor_get(x_14, 0); lean_inc(x_60); lean_dec(x_14); x_61 = lean_box(0); -x_62 = l_Lean_Language_Lean_process_parseCmd(x_61, x_11, x_58, x_60, x_10, x_59); -return x_62; +x_62 = 0; +x_63 = l_Lean_Language_Lean_process_parseCmd(x_61, x_11, x_58, x_60, x_62, x_10, x_59); +return x_63; } } else { -uint8_t x_63; +uint8_t x_64; lean_dec(x_14); lean_dec(x_11); lean_dec(x_10); -x_63 = !lean_is_exclusive(x_51); -if (x_63 == 0) +x_64 = !lean_is_exclusive(x_51); +if (x_64 == 0) { return x_51; } else { -lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_64 = lean_ctor_get(x_51, 0); -x_65 = lean_ctor_get(x_51, 1); +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_inc(x_64); lean_dec(x_51); -x_66 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_66, 0, x_64); -lean_ctor_set(x_66, 1, x_65); -return x_66; +x_67 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_67, 0, x_65); +lean_ctor_set(x_67, 1, x_66); +return x_67; } } } else { -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_43, 0); -lean_inc(x_67); -lean_dec(x_43); -x_68 = lean_ctor_get(x_67, 1); +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_68 = lean_ctor_get(x_43, 0); lean_inc(x_68); -x_69 = lean_ctor_get(x_67, 3); +lean_dec(x_43); +x_69 = lean_ctor_get(x_68, 1); lean_inc(x_69); -lean_dec(x_67); -x_70 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_70, 0, x_68); -lean_ctor_set(x_70, 1, x_69); -lean_ctor_set(x_3, 0, x_70); +x_70 = lean_ctor_get(x_68, 3); +lean_inc(x_70); +lean_dec(x_68); x_71 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_71, 0, x_3); -lean_ctor_set(x_71, 1, x_4); +lean_ctor_set(x_71, 0, x_69); +lean_ctor_set(x_71, 1, x_70); +lean_ctor_set(x_3, 0, x_71); +x_72 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_72, 0, x_3); +lean_ctor_set(x_72, 1, x_4); lean_inc(x_10); -x_72 = l_Lean_Language_Lean_process_doElab(x_5, x_6, x_7, x_71, x_8, x_9, x_10, x_44); +x_73 = l_Lean_Language_Lean_process_doElab(x_5, x_6, x_7, x_72, x_8, x_9, x_10, x_44); lean_dec(x_9); -if (lean_obj_tag(x_72) == 0) +if (lean_obj_tag(x_73) == 0) { if (lean_obj_tag(x_14) == 0) { -lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; +lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_dec(x_11); lean_dec(x_10); -x_73 = lean_ctor_get(x_72, 1); -lean_inc(x_73); -if (lean_is_exclusive(x_72)) { - lean_ctor_release(x_72, 0); - lean_ctor_release(x_72, 1); - x_74 = x_72; +x_74 = lean_ctor_get(x_73, 1); +lean_inc(x_74); +if (lean_is_exclusive(x_73)) { + lean_ctor_release(x_73, 0); + lean_ctor_release(x_73, 1); + x_75 = x_73; } else { - lean_dec_ref(x_72); - x_74 = lean_box(0); + lean_dec_ref(x_73); + x_75 = lean_box(0); } -x_75 = lean_box(0); -if (lean_is_scalar(x_74)) { - x_76 = lean_alloc_ctor(0, 2, 0); +x_76 = lean_box(0); +if (lean_is_scalar(x_75)) { + x_77 = lean_alloc_ctor(0, 2, 0); } else { - x_76 = x_74; + x_77 = x_75; } -lean_ctor_set(x_76, 0, x_75); -lean_ctor_set(x_76, 1, x_73); -return x_76; +lean_ctor_set(x_77, 0, x_76); +lean_ctor_set(x_77, 1, x_74); +return x_77; } else { -lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; -x_77 = lean_ctor_get(x_72, 0); -lean_inc(x_77); -x_78 = lean_ctor_get(x_72, 1); +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_78 = lean_ctor_get(x_73, 0); lean_inc(x_78); -lean_dec(x_72); -x_79 = lean_ctor_get(x_14, 0); +x_79 = lean_ctor_get(x_73, 1); lean_inc(x_79); +lean_dec(x_73); +x_80 = lean_ctor_get(x_14, 0); +lean_inc(x_80); lean_dec(x_14); -x_80 = lean_box(0); -x_81 = l_Lean_Language_Lean_process_parseCmd(x_80, x_11, x_77, x_79, x_10, x_78); -return x_81; +x_81 = lean_box(0); +x_82 = 0; +x_83 = l_Lean_Language_Lean_process_parseCmd(x_81, x_11, x_78, x_80, x_82, x_10, x_79); +return x_83; } } else { -lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; +lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_dec(x_14); lean_dec(x_11); lean_dec(x_10); -x_82 = lean_ctor_get(x_72, 0); -lean_inc(x_82); -x_83 = lean_ctor_get(x_72, 1); -lean_inc(x_83); -if (lean_is_exclusive(x_72)) { - lean_ctor_release(x_72, 0); - lean_ctor_release(x_72, 1); - x_84 = x_72; +x_84 = lean_ctor_get(x_73, 0); +lean_inc(x_84); +x_85 = lean_ctor_get(x_73, 1); +lean_inc(x_85); +if (lean_is_exclusive(x_73)) { + lean_ctor_release(x_73, 0); + lean_ctor_release(x_73, 1); + x_86 = x_73; } else { - lean_dec_ref(x_72); - x_84 = lean_box(0); + lean_dec_ref(x_73); + x_86 = lean_box(0); } -if (lean_is_scalar(x_84)) { - x_85 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_86)) { + x_87 = lean_alloc_ctor(1, 2, 0); } else { - x_85 = x_84; + x_87 = x_86; } -lean_ctor_set(x_85, 0, x_82); -lean_ctor_set(x_85, 1, x_83); -return x_85; +lean_ctor_set(x_87, 0, x_84); +lean_ctor_set(x_87, 1, x_85); +return x_87; } } } 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; -x_86 = lean_ctor_get(x_3, 0); -lean_inc(x_86); -lean_dec(x_3); -x_87 = lean_ctor_get(x_23, 1); -lean_inc(x_87); -lean_dec(x_23); -x_88 = lean_ctor_get(x_86, 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; +x_88 = lean_ctor_get(x_3, 0); lean_inc(x_88); -if (lean_is_exclusive(x_86)) { - lean_ctor_release(x_86, 0); - lean_ctor_release(x_86, 1); - x_89 = x_86; +lean_dec(x_3); +x_89 = lean_ctor_get(x_22, 1); +lean_inc(x_89); +lean_dec(x_22); +x_90 = lean_ctor_get(x_88, 0); +lean_inc(x_90); +if (lean_is_exclusive(x_88)) { + lean_ctor_release(x_88, 0); + lean_ctor_release(x_88, 1); + x_91 = x_88; } else { - lean_dec_ref(x_86); - x_89 = lean_box(0); + lean_dec_ref(x_88); + x_91 = lean_box(0); } -x_90 = lean_ctor_get(x_88, 1); -lean_inc(x_90); -x_91 = lean_ctor_get(x_88, 3); -lean_inc(x_91); -lean_dec(x_88); -if (lean_is_scalar(x_89)) { - x_92 = lean_alloc_ctor(0, 2, 0); +x_92 = lean_ctor_get(x_90, 1); +lean_inc(x_92); +x_93 = lean_ctor_get(x_90, 3); +lean_inc(x_93); +lean_dec(x_90); +if (lean_is_scalar(x_91)) { + x_94 = lean_alloc_ctor(0, 2, 0); } else { - x_92 = x_89; + x_94 = x_91; } -lean_ctor_set(x_92, 0, x_90); -lean_ctor_set(x_92, 1, x_91); -x_93 = lean_alloc_ctor(1, 1, 0); -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_4); +lean_ctor_set(x_94, 0, x_92); +lean_ctor_set(x_94, 1, x_93); +x_95 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_95, 0, x_94); +x_96 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_96, 0, x_95); +lean_ctor_set(x_96, 1, x_4); lean_inc(x_10); -x_95 = l_Lean_Language_Lean_process_doElab(x_5, x_6, x_7, x_94, x_8, x_9, x_10, x_87); +x_97 = l_Lean_Language_Lean_process_doElab(x_5, x_6, x_7, x_96, x_8, x_9, x_10, x_89); lean_dec(x_9); -if (lean_obj_tag(x_95) == 0) +if (lean_obj_tag(x_97) == 0) { if (lean_obj_tag(x_14) == 0) { -lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; +lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_dec(x_11); lean_dec(x_10); -x_96 = lean_ctor_get(x_95, 1); -lean_inc(x_96); -if (lean_is_exclusive(x_95)) { - lean_ctor_release(x_95, 0); - lean_ctor_release(x_95, 1); - x_97 = x_95; +x_98 = lean_ctor_get(x_97, 1); +lean_inc(x_98); +if (lean_is_exclusive(x_97)) { + lean_ctor_release(x_97, 0); + lean_ctor_release(x_97, 1); + x_99 = x_97; } else { - lean_dec_ref(x_95); - x_97 = lean_box(0); + lean_dec_ref(x_97); + x_99 = lean_box(0); } -x_98 = lean_box(0); -if (lean_is_scalar(x_97)) { - x_99 = lean_alloc_ctor(0, 2, 0); +x_100 = lean_box(0); +if (lean_is_scalar(x_99)) { + x_101 = lean_alloc_ctor(0, 2, 0); } else { - x_99 = x_97; + x_101 = x_99; } -lean_ctor_set(x_99, 0, x_98); -lean_ctor_set(x_99, 1, x_96); -return x_99; +lean_ctor_set(x_101, 0, x_100); +lean_ctor_set(x_101, 1, x_98); +return x_101; } else { -lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; -x_100 = lean_ctor_get(x_95, 0); -lean_inc(x_100); -x_101 = lean_ctor_get(x_95, 1); -lean_inc(x_101); -lean_dec(x_95); -x_102 = lean_ctor_get(x_14, 0); +lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; uint8_t x_106; lean_object* x_107; +x_102 = lean_ctor_get(x_97, 0); lean_inc(x_102); +x_103 = lean_ctor_get(x_97, 1); +lean_inc(x_103); +lean_dec(x_97); +x_104 = lean_ctor_get(x_14, 0); +lean_inc(x_104); lean_dec(x_14); -x_103 = lean_box(0); -x_104 = l_Lean_Language_Lean_process_parseCmd(x_103, x_11, x_100, x_102, x_10, x_101); -return x_104; +x_105 = lean_box(0); +x_106 = 0; +x_107 = l_Lean_Language_Lean_process_parseCmd(x_105, x_11, x_102, x_104, x_106, x_10, x_103); +return x_107; } } else { -lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; +lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_dec(x_14); lean_dec(x_11); lean_dec(x_10); -x_105 = lean_ctor_get(x_95, 0); -lean_inc(x_105); -x_106 = lean_ctor_get(x_95, 1); -lean_inc(x_106); -if (lean_is_exclusive(x_95)) { - lean_ctor_release(x_95, 0); - lean_ctor_release(x_95, 1); - x_107 = x_95; +x_108 = lean_ctor_get(x_97, 0); +lean_inc(x_108); +x_109 = lean_ctor_get(x_97, 1); +lean_inc(x_109); +if (lean_is_exclusive(x_97)) { + lean_ctor_release(x_97, 0); + lean_ctor_release(x_97, 1); + x_110 = x_97; } else { - lean_dec_ref(x_95); - x_107 = lean_box(0); + lean_dec_ref(x_97); + x_110 = lean_box(0); } -if (lean_is_scalar(x_107)) { - x_108 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_110)) { + x_111 = lean_alloc_ctor(1, 2, 0); } else { - x_108 = x_107; + x_111 = x_110; } -lean_ctor_set(x_108, 0, x_105); -lean_ctor_set(x_108, 1, x_106); -return x_108; +lean_ctor_set(x_111, 0, x_108); +lean_ctor_set(x_111, 1, x_109); +return x_111; } } } } else { -uint8_t x_109; +uint8_t x_112; lean_dec(x_14); lean_dec(x_11); lean_dec(x_10); @@ -5134,23 +5144,23 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_109 = !lean_is_exclusive(x_23); -if (x_109 == 0) +x_112 = !lean_is_exclusive(x_22); +if (x_112 == 0) { -return x_23; +return x_22; } else { -lean_object* x_110; lean_object* x_111; lean_object* x_112; -x_110 = lean_ctor_get(x_23, 0); -x_111 = lean_ctor_get(x_23, 1); -lean_inc(x_111); -lean_inc(x_110); -lean_dec(x_23); -x_112 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_112, 0, x_110); -lean_ctor_set(x_112, 1, x_111); -return x_112; +lean_object* x_113; lean_object* x_114; lean_object* x_115; +x_113 = lean_ctor_get(x_22, 0); +x_114 = lean_ctor_get(x_22, 1); +lean_inc(x_114); +lean_inc(x_113); +lean_dec(x_22); +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; } } } @@ -5158,7 +5168,7 @@ return x_112; } else { -uint8_t x_153; +uint8_t x_156; lean_dec(x_14); lean_dec(x_13); lean_dec(x_11); @@ -5169,23 +5179,23 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_153 = !lean_is_exclusive(x_17); -if (x_153 == 0) +x_156 = !lean_is_exclusive(x_16); +if (x_156 == 0) { -return x_17; +return x_16; } else { -lean_object* x_154; lean_object* x_155; lean_object* x_156; -x_154 = lean_ctor_get(x_17, 0); -x_155 = lean_ctor_get(x_17, 1); -lean_inc(x_155); -lean_inc(x_154); -lean_dec(x_17); -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_157; lean_object* x_158; lean_object* x_159; +x_157 = lean_ctor_get(x_16, 0); +x_158 = lean_ctor_get(x_16, 1); +lean_inc(x_158); +lean_inc(x_157); +lean_dec(x_16); +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; } } } @@ -5201,173 +5211,164 @@ lean_ctor_set(x_2, 1, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___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_Language_Lean_process_parseCmd___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_13; -x_13 = lean_io_promise_new(x_12); -if (lean_obj_tag(x_13) == 0) +lean_object* x_12; +x_12 = lean_io_promise_new(x_11); +if (lean_obj_tag(x_12) == 0) { -lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_14 = lean_ctor_get(x_13, 0); +lean_object* x_13; lean_object* x_14; uint8_t 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); -x_15 = lean_ctor_get(x_13, 1); -lean_inc(x_15); -lean_dec(x_13); -x_16 = lean_io_promise_new(x_15); +lean_dec(x_12); +x_15 = 0; +x_16 = l_Lean_Syntax_getTailPos_x3f(x_1, x_15); +lean_inc(x_13); +x_17 = lean_io_promise_result(x_13); if (lean_obj_tag(x_16) == 0) { -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 = 0; -x_20 = l_Lean_Syntax_getTailPos_x3f(x_1, x_19); -lean_inc(x_17); -x_21 = lean_io_promise_result(x_17); -if (lean_obj_tag(x_20) == 0) -{ -lean_object* x_53; -x_53 = lean_box(0); -x_22 = x_53; -goto block_52; +lean_object* x_49; +x_49 = lean_box(0); +x_18 = x_49; +goto block_48; } else { -uint8_t x_54; -x_54 = !lean_is_exclusive(x_20); -if (x_54 == 0) +uint8_t x_50; +x_50 = !lean_is_exclusive(x_16); +if (x_50 == 0) { -lean_object* x_55; lean_object* x_56; -x_55 = lean_ctor_get(x_20, 0); -lean_inc(x_55); -x_56 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_56, 0, x_55); -lean_ctor_set(x_56, 1, x_55); -lean_ctor_set(x_20, 0, x_56); -x_22 = x_20; -goto block_52; +lean_object* x_51; lean_object* x_52; +x_51 = lean_ctor_get(x_16, 0); +lean_inc(x_51); +x_52 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_52, 0, x_51); +lean_ctor_set(x_52, 1, x_51); +lean_ctor_set(x_16, 0, x_52); +x_18 = x_16; +goto block_48; } else { -lean_object* x_57; lean_object* x_58; lean_object* x_59; -x_57 = lean_ctor_get(x_20, 0); -lean_inc(x_57); -lean_dec(x_20); -lean_inc(x_57); -x_58 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_58, 0, x_57); -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_22 = x_59; -goto block_52; +lean_object* x_53; lean_object* x_54; lean_object* x_55; +x_53 = lean_ctor_get(x_16, 0); +lean_inc(x_53); +lean_dec(x_16); +lean_inc(x_53); +x_54 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_54, 0, x_53); +lean_ctor_set(x_54, 1, x_53); +x_55 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_55, 0, x_54); +x_18 = x_55; +goto block_48; } } -block_52: +block_48: { -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_23, 0, x_22); -lean_ctor_set(x_23, 1, x_21); +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set(x_19, 1, x_17); if (lean_obj_tag(x_5) == 0) { -lean_object* x_41; lean_object* x_42; -x_41 = l_Lean_Language_Lean_process_parseCmd___lambda__3___closed__1; -x_42 = lean_st_mk_ref(x_41, x_18); -if (lean_obj_tag(x_42) == 0) +lean_object* x_37; lean_object* x_38; +x_37 = l_Lean_Language_Lean_process_parseCmd___lambda__3___closed__1; +x_38 = lean_st_mk_ref(x_37, x_14); +if (lean_obj_tag(x_38) == 0) { -lean_object* x_43; lean_object* x_44; -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_24 = x_43; -x_25 = x_44; -goto block_40; +lean_object* x_39; lean_object* x_40; +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_20 = x_39; +x_21 = x_40; +goto block_36; } else { -uint8_t x_45; -lean_dec(x_23); -lean_dec(x_17); -lean_dec(x_14); +uint8_t x_41; +lean_dec(x_19); +lean_dec(x_13); +lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_3); lean_dec(x_1); -x_45 = !lean_is_exclusive(x_42); -if (x_45 == 0) +x_41 = !lean_is_exclusive(x_38); +if (x_41 == 0) { -return x_42; +return x_38; } else { -lean_object* x_46; lean_object* x_47; lean_object* x_48; -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_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_42; lean_object* x_43; lean_object* x_44; +x_42 = lean_ctor_get(x_38, 0); +x_43 = lean_ctor_get(x_38, 1); +lean_inc(x_43); +lean_inc(x_42); +lean_dec(x_38); +x_44 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_44, 0, x_42); +lean_ctor_set(x_44, 1, x_43); +return x_44; } } } else { -lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_49 = lean_ctor_get(x_5, 0); -lean_inc(x_49); -x_50 = lean_ctor_get(x_49, 0); -lean_inc(x_50); -lean_dec(x_49); -x_51 = lean_ctor_get(x_50, 5); -lean_inc(x_51); -lean_dec(x_50); -x_24 = x_51; -x_25 = x_18; -goto block_40; +lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_45 = lean_ctor_get(x_5, 0); +lean_inc(x_45); +x_46 = lean_ctor_get(x_45, 0); +lean_inc(x_46); +lean_dec(x_45); +x_47 = lean_ctor_get(x_46, 5); +lean_inc(x_47); +lean_dec(x_46); +x_20 = x_47; +x_21 = x_14; +goto block_36; } -block_40: +block_36: { -lean_object* x_26; uint8_t x_27; uint8_t x_28; -x_26 = l_Lean_Language_Lean_process_doElab___closed__1; -x_27 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_2, x_26); +lean_object* x_22; uint8_t x_23; uint8_t x_24; +x_22 = l_Lean_Language_Lean_process_doElab___closed__1; +x_23 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_2, x_22); lean_inc(x_1); -x_28 = l_Lean_Parser_isTerminalCommand(x_1); -if (x_28 == 0) +x_24 = l_Lean_Parser_isTerminalCommand(x_1); +if (x_24 == 0) { -lean_object* x_29; -x_29 = lean_io_promise_new(x_25); -if (lean_obj_tag(x_29) == 0) +lean_object* x_25; +x_25 = lean_io_promise_new(x_21); +if (lean_obj_tag(x_25) == 0) { -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_30 = lean_ctor_get(x_29, 0); -lean_inc(x_30); -x_31 = lean_ctor_get(x_29, 1); -lean_inc(x_31); -lean_dec(x_29); -x_32 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_32, 0, x_30); -x_33 = l_Lean_Language_Lean_process_parseCmd___lambda__2(x_3, x_4, x_5, x_14, x_1, x_6, x_7, x_17, x_24, x_8, x_9, x_27, x_23, x_32, x_11, x_31); -lean_dec(x_17); -return x_33; +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_26 = lean_ctor_get(x_25, 0); +lean_inc(x_26); +x_27 = lean_ctor_get(x_25, 1); +lean_inc(x_27); +lean_dec(x_25); +x_28 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_28, 0, x_26); +x_29 = l_Lean_Language_Lean_process_parseCmd___lambda__2(x_3, x_4, x_5, x_10, x_1, x_6, x_7, x_13, x_20, x_8, x_9, x_23, x_19, x_28, x_27); +lean_dec(x_13); +return x_29; } else { -uint8_t x_34; -lean_dec(x_24); -lean_dec(x_23); -lean_dec(x_17); -lean_dec(x_14); +uint8_t x_30; +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_13); +lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -5375,41 +5376,41 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); lean_dec(x_1); -x_34 = !lean_is_exclusive(x_29); -if (x_34 == 0) +x_30 = !lean_is_exclusive(x_25); +if (x_30 == 0) { -return x_29; +return x_25; } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_35 = lean_ctor_get(x_29, 0); -x_36 = lean_ctor_get(x_29, 1); -lean_inc(x_36); -lean_inc(x_35); -lean_dec(x_29); -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_31; lean_object* x_32; lean_object* x_33; +x_31 = lean_ctor_get(x_25, 0); +x_32 = lean_ctor_get(x_25, 1); +lean_inc(x_32); +lean_inc(x_31); +lean_dec(x_25); +x_33 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_33, 0, x_31); +lean_ctor_set(x_33, 1, x_32); +return x_33; } } } else { -lean_object* x_38; lean_object* x_39; -x_38 = lean_box(0); -x_39 = l_Lean_Language_Lean_process_parseCmd___lambda__2(x_3, x_4, x_5, x_14, x_1, x_6, x_7, x_17, x_24, x_8, x_9, x_27, x_23, x_38, x_11, x_25); -lean_dec(x_17); -return x_39; +lean_object* x_34; lean_object* x_35; +x_34 = lean_box(0); +x_35 = l_Lean_Language_Lean_process_parseCmd___lambda__2(x_3, x_4, x_5, x_10, x_1, x_6, x_7, x_13, x_20, x_8, x_9, x_23, x_19, x_34, x_21); +lean_dec(x_13); +return x_35; } } } } else { -uint8_t x_60; -lean_dec(x_14); +uint8_t x_56; +lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -5417,361 +5418,278 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); lean_dec(x_1); -x_60 = !lean_is_exclusive(x_16); -if (x_60 == 0) +x_56 = !lean_is_exclusive(x_12); +if (x_56 == 0) { -return x_16; +return x_12; } else { -lean_object* x_61; lean_object* x_62; lean_object* x_63; -x_61 = lean_ctor_get(x_16, 0); -x_62 = lean_ctor_get(x_16, 1); -lean_inc(x_62); -lean_inc(x_61); -lean_dec(x_16); -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; +lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_57 = lean_ctor_get(x_12, 0); +x_58 = lean_ctor_get(x_12, 1); +lean_inc(x_58); +lean_inc(x_57); +lean_dec(x_12); +x_59 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_59, 0, x_57); +lean_ctor_set(x_59, 1, x_58); +return x_59; } } } -else -{ -uint8_t x_64; -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -lean_dec(x_1); -x_64 = !lean_is_exclusive(x_13); -if (x_64 == 0) -{ -return x_13; } -else +static lean_object* _init_l_Lean_Language_Lean_process_parseCmd___lambda__4___closed__1() { +_start: { -lean_object* x_65; lean_object* x_66; lean_object* x_67; -x_65 = lean_ctor_get(x_13, 0); -x_66 = lean_ctor_get(x_13, 1); -lean_inc(x_66); -lean_inc(x_65); -lean_dec(x_13); -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_1; +x_1 = lean_alloc_closure((void*)(l_IO_Promise_new___boxed), 3, 2); +lean_closure_set(x_1, 0, lean_box(0)); +lean_closure_set(x_1, 1, lean_box(0)); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___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_Language_Lean_process_parseCmd___lambda__4(uint8_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -lean_object* x_6; -x_6 = lean_ctor_get(x_1, 2); -if (lean_obj_tag(x_6) == 0) +if (x_1 == 0) { -lean_object* x_7; lean_object* x_8; -x_7 = lean_box(0); -x_8 = lean_apply_3(x_2, x_7, x_4, x_5); -return x_8; -} -else +lean_object* x_14; +x_14 = lean_io_promise_new(x_13); +if (lean_obj_tag(x_14) == 0) { -lean_object* x_9; uint8_t x_10; lean_object* x_11; lean_object* x_12; -x_9 = lean_ctor_get(x_6, 0); -x_10 = 1; -x_11 = lean_box(x_10); -x_12 = lean_st_ref_set(x_9, x_11, x_5); -if (lean_obj_tag(x_12) == 0) +lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); +x_17 = lean_io_promise_new(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_inc(x_14); -lean_dec(x_12); -x_15 = lean_apply_3(x_2, x_13, x_4, x_14); -return x_15; +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_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_Syntax_getTailPos_x3f(x_2, x_20); +lean_inc(x_18); +x_22 = lean_io_promise_result(x_18); +if (lean_obj_tag(x_21) == 0) +{ +lean_object* x_74; +x_74 = lean_box(0); +x_23 = x_74; +goto block_73; } else { -uint8_t x_16; -lean_dec(x_4); -lean_dec(x_2); -x_16 = !lean_is_exclusive(x_12); -if (x_16 == 0) +uint8_t x_75; +x_75 = !lean_is_exclusive(x_21); +if (x_75 == 0) { -return x_12; +lean_object* x_76; lean_object* x_77; +x_76 = lean_ctor_get(x_21, 0); +lean_inc(x_76); +x_77 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_77, 0, x_76); +lean_ctor_set(x_77, 1, x_76); +lean_ctor_set(x_21, 0, x_77); +x_23 = x_21; +goto block_73; } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_12, 0); -x_18 = lean_ctor_get(x_12, 1); -lean_inc(x_18); -lean_inc(x_17); -lean_dec(x_12); -x_19 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_19, 0, x_17); -lean_ctor_set(x_19, 1, x_18); -return x_19; -} -} -} -} -} -static lean_object* _init_l_Lean_Language_Lean_process_parseCmd___lambda__5___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = lean_box(0); -x_2 = l_Lean_Language_SnapshotTask_pure___rarg(x_1); -return x_2; +lean_object* x_78; lean_object* x_79; lean_object* x_80; +x_78 = lean_ctor_get(x_21, 0); +lean_inc(x_78); +lean_dec(x_21); +lean_inc(x_78); +x_79 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_79, 0, x_78); +lean_ctor_set(x_79, 1, x_78); +x_80 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_80, 0, x_79); +x_23 = x_80; +goto block_73; } } -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___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: +block_73: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; -x_7 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_7, 0, x_5); -x_8 = lean_ctor_get(x_1, 1); -lean_inc(x_8); -lean_dec(x_1); -x_9 = l_Lean_Language_Lean_process_parseCmd(x_7, x_2, x_8, x_3, x_4, x_6); -if (lean_obj_tag(x_9) == 0) +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_23); +lean_ctor_set(x_24, 1, x_22); +if (lean_obj_tag(x_6) == 0) { -uint8_t x_10; -x_10 = !lean_is_exclusive(x_9); -if (x_10 == 0) +lean_object* x_62; lean_object* x_63; +x_62 = l_Lean_Language_Lean_process_parseCmd___lambda__3___closed__1; +x_63 = lean_st_mk_ref(x_62, x_19); +if (lean_obj_tag(x_63) == 0) { -lean_object* x_11; lean_object* x_12; -x_11 = lean_ctor_get(x_9, 0); -lean_dec(x_11); -x_12 = l_Lean_Language_Lean_process_parseCmd___lambda__5___closed__1; -lean_ctor_set(x_9, 0, x_12); -return x_9; +lean_object* x_64; lean_object* x_65; +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_25 = x_64; +x_26 = x_65; +goto block_61; } else { -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_ctor_get(x_9, 1); -lean_inc(x_13); +uint8_t x_66; +lean_dec(x_24); +lean_dec(x_18); +lean_dec(x_15); +lean_dec(x_10); lean_dec(x_9); -x_14 = l_Lean_Language_Lean_process_parseCmd___lambda__5___closed__1; -x_15 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_15, 0, x_14); -lean_ctor_set(x_15, 1, x_13); -return x_15; -} -} -else -{ -uint8_t x_16; -x_16 = !lean_is_exclusive(x_9); -if (x_16 == 0) +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_66 = !lean_is_exclusive(x_63); +if (x_66 == 0) { -return x_9; +return x_63; } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_9, 0); -x_18 = lean_ctor_get(x_9, 1); -lean_inc(x_18); -lean_inc(x_17); -lean_dec(x_9); -x_19 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_19, 0, x_17); -lean_ctor_set(x_19, 1, x_18); -return x_19; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___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; uint8_t x_9; lean_object* x_10; -x_7 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_parseCmd___lambda__5), 6, 4); -lean_closure_set(x_7, 0, x_5); -lean_closure_set(x_7, 1, x_1); -lean_closure_set(x_7, 2, x_2); -lean_closure_set(x_7, 3, x_3); -x_8 = lean_ctor_get(x_4, 0); -lean_inc(x_8); -x_9 = 1; -x_10 = l_Lean_Language_SnapshotTask_bindIO___rarg(x_4, x_7, x_8, x_9, x_6); -return x_10; -} +lean_object* x_67; lean_object* x_68; lean_object* x_69; +x_67 = lean_ctor_get(x_63, 0); +x_68 = lean_ctor_get(x_63, 1); +lean_inc(x_68); +lean_inc(x_67); +lean_dec(x_63); +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; } -static lean_object* _init_l_Lean_Language_Lean_process_parseCmd___lambda__7___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("parsing", 7, 7); -return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___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: -{ -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; 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_9 = lean_ctor_get(x_1, 0); -lean_inc(x_9); -x_10 = lean_ctor_get(x_2, 0); -lean_inc(x_10); -x_11 = lean_ctor_get(x_2, 2); -lean_inc(x_11); -x_12 = l_Lean_Elab_Command_instInhabitedScope; -x_13 = l_List_head_x21___rarg(x_12, x_11); -lean_dec(x_11); -x_14 = lean_ctor_get(x_13, 1); -lean_inc(x_14); -x_15 = lean_ctor_get(x_13, 2); -lean_inc(x_15); -x_16 = lean_ctor_get(x_13, 3); -lean_inc(x_16); -lean_dec(x_13); -lean_inc(x_14); -x_17 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_17, 0, x_10); -lean_ctor_set(x_17, 1, x_14); -lean_ctor_set(x_17, 2, x_15); -lean_ctor_set(x_17, 3, x_16); -lean_inc(x_3); -x_18 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_parseCmd___lambda__1___boxed), 4, 3); -lean_closure_set(x_18, 0, x_3); -lean_closure_set(x_18, 1, x_17); -lean_closure_set(x_18, 2, x_1); -x_19 = l_Lean_Language_Lean_process_parseCmd___lambda__7___closed__1; -x_20 = lean_box(0); -x_21 = lean_profileit(x_19, x_14, x_18, x_20); -x_22 = lean_ctor_get(x_21, 1); -lean_inc(x_22); -if (lean_obj_tag(x_5) == 0) +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_21, 0); -lean_inc(x_23); -lean_dec(x_21); -x_24 = lean_ctor_get(x_22, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_22, 1); -lean_inc(x_25); -lean_dec(x_22); -x_26 = lean_box(0); -x_27 = l_Lean_Language_Lean_process_parseCmd___lambda__3(x_23, x_14, x_25, x_4, x_5, x_2, x_9, x_3, x_24, x_26, x_7, x_8); -lean_dec(x_7); -lean_dec(x_4); -lean_dec(x_14); -return x_27; +lean_object* x_70; lean_object* x_71; lean_object* x_72; +x_70 = lean_ctor_get(x_6, 0); +lean_inc(x_70); +x_71 = lean_ctor_get(x_70, 0); +lean_inc(x_71); +lean_dec(x_70); +x_72 = lean_ctor_get(x_71, 5); +lean_inc(x_72); +lean_dec(x_71); +x_25 = x_72; +x_26 = x_19; +goto block_61; } -else +block_61: { -lean_object* x_28; uint8_t x_29; -x_28 = lean_ctor_get(x_21, 0); -lean_inc(x_28); -lean_dec(x_21); -x_29 = !lean_is_exclusive(x_22); +lean_object* x_27; uint8_t x_28; uint8_t x_29; +x_27 = l_Lean_Language_Lean_process_doElab___closed__1; +x_28 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_3, x_27); +lean_dec(x_3); +lean_inc(x_2); +x_29 = l_Lean_Parser_isTerminalCommand(x_2); 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; uint8_t x_37; -x_30 = lean_ctor_get(x_22, 0); -x_31 = lean_ctor_get(x_22, 1); -x_32 = lean_ctor_get(x_5, 0); -lean_inc(x_32); -lean_inc(x_30); -lean_inc(x_3); -lean_inc(x_4); -lean_inc(x_28); -x_33 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_parseCmd___lambda__3___boxed), 12, 9); -lean_closure_set(x_33, 0, x_28); -lean_closure_set(x_33, 1, x_14); -lean_closure_set(x_33, 2, x_31); -lean_closure_set(x_33, 3, x_4); -lean_closure_set(x_33, 4, x_5); -lean_closure_set(x_33, 5, x_2); -lean_closure_set(x_33, 6, x_9); -lean_closure_set(x_33, 7, x_3); -lean_closure_set(x_33, 8, x_30); -x_34 = lean_ctor_get(x_32, 0); -lean_inc(x_34); -x_35 = lean_ctor_get(x_32, 1); -lean_inc(x_35); -x_36 = lean_ctor_get(x_34, 1); -lean_inc(x_36); -x_37 = l_Lean_Syntax_eqWithInfo(x_28, x_36); -if (x_37 == 0) +lean_object* x_30; +x_30 = lean_io_promise_new(x_26); +if (lean_obj_tag(x_30) == 0) { -lean_object* x_38; lean_object* x_39; -lean_dec(x_35); -lean_dec(x_34); -lean_dec(x_32); -lean_free_object(x_22); +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_31 = lean_ctor_get(x_30, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_30, 1); +lean_inc(x_32); lean_dec(x_30); -lean_dec(x_4); -x_38 = lean_box(0); -x_39 = l_Lean_Language_Lean_process_parseCmd___lambda__4(x_3, x_33, x_38, x_7, x_8); -lean_dec(x_3); -return x_39; +x_33 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_33, 0, x_31); +x_34 = l_Lean_Language_Lean_process_parseCmd___lambda__2(x_4, x_5, x_6, x_15, x_2, x_7, x_8, x_18, x_25, x_9, x_10, x_28, x_24, x_33, x_32); +lean_dec(x_18); +lean_dec(x_5); +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; lean_object* x_37; +x_36 = lean_ctor_get(x_34, 0); +lean_dec(x_36); +x_37 = lean_box(0); +lean_ctor_set(x_34, 0, x_37); +return x_34; } else { -lean_dec(x_33); -lean_dec(x_7); -if (lean_obj_tag(x_35) == 0) -{ -lean_object* x_40; +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_34, 1); +lean_inc(x_38); lean_dec(x_34); -lean_free_object(x_22); -lean_dec(x_30); -lean_dec(x_3); -x_40 = lean_io_promise_resolve(x_32, x_4, x_8); -lean_dec(x_4); -if (lean_obj_tag(x_40) == 0) +x_39 = lean_box(0); +x_40 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_40, 0, x_39); +lean_ctor_set(x_40, 1, x_38); +return x_40; +} +} +else { uint8_t x_41; -x_41 = !lean_is_exclusive(x_40); +x_41 = !lean_is_exclusive(x_34); if (x_41 == 0) { -return x_40; +return x_34; } 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); +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_40); -x_44 = lean_alloc_ctor(0, 2, 0); +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 { uint8_t x_45; -x_45 = !lean_is_exclusive(x_40); +lean_dec(x_25); +lean_dec(x_24); +lean_dec(x_18); +lean_dec(x_15); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +x_45 = !lean_is_exclusive(x_30); if (x_45 == 0) { -return x_40; +return x_30; } 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); +x_46 = lean_ctor_get(x_30, 0); +x_47 = lean_ctor_get(x_30, 1); lean_inc(x_47); lean_inc(x_46); -lean_dec(x_40); +lean_dec(x_30); x_48 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_48, 0, x_46); lean_ctor_set(x_48, 1, x_47); @@ -5781,242 +5699,940 @@ return x_48; } else { -uint8_t x_49; -x_49 = !lean_is_exclusive(x_32); -if (x_49 == 0) -{ -lean_object* x_50; lean_object* x_51; uint8_t x_52; -x_50 = lean_ctor_get(x_32, 1); -lean_dec(x_50); -x_51 = lean_ctor_get(x_32, 0); -lean_dec(x_51); -x_52 = !lean_is_exclusive(x_35); -if (x_52 == 0) -{ -lean_object* x_53; lean_object* x_54; -x_53 = lean_ctor_get(x_35, 0); -x_54 = lean_io_promise_new(x_8); -if (lean_obj_tag(x_54) == 0) -{ -lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; uint8_t x_60; lean_object* x_61; -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); -lean_inc(x_55); -x_57 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_parseCmd___lambda__6), 6, 4); -lean_closure_set(x_57, 0, x_30); -lean_closure_set(x_57, 1, x_55); -lean_closure_set(x_57, 2, x_3); -lean_closure_set(x_57, 3, x_53); -x_58 = lean_ctor_get(x_34, 4); -lean_inc(x_58); -x_59 = lean_ctor_get(x_58, 0); -lean_inc(x_59); -x_60 = 0; -x_61 = l_Lean_Language_SnapshotTask_bindIO___rarg(x_58, x_57, x_59, x_60, x_56); -if (lean_obj_tag(x_61) == 0) -{ -lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; -x_62 = lean_ctor_get(x_61, 1); -lean_inc(x_62); -lean_dec(x_61); -x_63 = lean_box(0); -x_64 = lean_io_promise_result(x_55); -lean_ctor_set(x_22, 1, x_64); -lean_ctor_set(x_22, 0, x_63); -lean_ctor_set(x_35, 0, x_22); -x_65 = lean_io_promise_resolve(x_32, x_4, x_62); -lean_dec(x_4); -if (lean_obj_tag(x_65) == 0) +lean_object* x_49; lean_object* x_50; +x_49 = lean_box(0); +x_50 = l_Lean_Language_Lean_process_parseCmd___lambda__2(x_4, x_5, x_6, x_15, x_2, x_7, x_8, x_18, x_25, x_9, x_10, x_28, x_24, x_49, x_26); +lean_dec(x_18); +lean_dec(x_5); +if (lean_obj_tag(x_50) == 0) { -uint8_t x_66; -x_66 = !lean_is_exclusive(x_65); -if (x_66 == 0) +uint8_t x_51; +x_51 = !lean_is_exclusive(x_50); +if (x_51 == 0) { -return x_65; +lean_object* x_52; lean_object* x_53; +x_52 = lean_ctor_get(x_50, 0); +lean_dec(x_52); +x_53 = lean_box(0); +lean_ctor_set(x_50, 0, x_53); +return x_50; } else { -lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_67 = lean_ctor_get(x_65, 0); -x_68 = lean_ctor_get(x_65, 1); -lean_inc(x_68); -lean_inc(x_67); -lean_dec(x_65); -x_69 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_69, 0, x_67); -lean_ctor_set(x_69, 1, x_68); -return x_69; +lean_object* x_54; lean_object* x_55; lean_object* x_56; +x_54 = lean_ctor_get(x_50, 1); +lean_inc(x_54); +lean_dec(x_50); +x_55 = lean_box(0); +x_56 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_56, 0, x_55); +lean_ctor_set(x_56, 1, x_54); +return x_56; } } else { -uint8_t x_70; -x_70 = !lean_is_exclusive(x_65); -if (x_70 == 0) +uint8_t x_57; +x_57 = !lean_is_exclusive(x_50); +if (x_57 == 0) { -return x_65; +return x_50; } else { -lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_71 = lean_ctor_get(x_65, 0); -x_72 = lean_ctor_get(x_65, 1); -lean_inc(x_72); -lean_inc(x_71); -lean_dec(x_65); -x_73 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_73, 0, x_71); -lean_ctor_set(x_73, 1, x_72); -return x_73; +lean_object* x_58; lean_object* x_59; lean_object* x_60; +x_58 = lean_ctor_get(x_50, 0); +x_59 = lean_ctor_get(x_50, 1); +lean_inc(x_59); +lean_inc(x_58); +lean_dec(x_50); +x_60 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_60, 0, x_58); +lean_ctor_set(x_60, 1, x_59); +return x_60; +} +} +} } } } else { -uint8_t x_74; -lean_dec(x_55); -lean_free_object(x_35); -lean_free_object(x_32); -lean_dec(x_34); -lean_free_object(x_22); +uint8_t x_81; +lean_dec(x_15); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); -x_74 = !lean_is_exclusive(x_61); -if (x_74 == 0) +lean_dec(x_3); +lean_dec(x_2); +x_81 = !lean_is_exclusive(x_17); +if (x_81 == 0) { -return x_61; +return x_17; } else { -lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_75 = lean_ctor_get(x_61, 0); -x_76 = lean_ctor_get(x_61, 1); -lean_inc(x_76); -lean_inc(x_75); -lean_dec(x_61); -x_77 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_77, 0, x_75); -lean_ctor_set(x_77, 1, x_76); -return x_77; +lean_object* x_82; lean_object* x_83; lean_object* x_84; +x_82 = lean_ctor_get(x_17, 0); +x_83 = lean_ctor_get(x_17, 1); +lean_inc(x_83); +lean_inc(x_82); +lean_dec(x_17); +x_84 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_84, 0, x_82); +lean_ctor_set(x_84, 1, x_83); +return x_84; +} +} +} +else +{ +uint8_t x_85; +lean_dec(x_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_85 = !lean_is_exclusive(x_14); +if (x_85 == 0) +{ +return x_14; +} +else +{ +lean_object* x_86; lean_object* x_87; lean_object* x_88; +x_86 = lean_ctor_get(x_14, 0); +x_87 = lean_ctor_get(x_14, 1); +lean_inc(x_87); +lean_inc(x_86); +lean_dec(x_14); +x_88 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_88, 0, x_86); +lean_ctor_set(x_88, 1, x_87); +return x_88; +} +} +} +else +{ +lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; +x_89 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_parseCmd___lambda__3___boxed), 11, 9); +lean_closure_set(x_89, 0, x_2); +lean_closure_set(x_89, 1, x_3); +lean_closure_set(x_89, 2, x_4); +lean_closure_set(x_89, 3, x_5); +lean_closure_set(x_89, 4, x_6); +lean_closure_set(x_89, 5, x_7); +lean_closure_set(x_89, 6, x_8); +lean_closure_set(x_89, 7, x_9); +lean_closure_set(x_89, 8, x_10); +x_90 = l_Lean_Language_Lean_process_parseCmd___lambda__4___closed__1; +x_91 = lean_alloc_closure((void*)(l_EStateM_bind___rarg), 3, 2); +lean_closure_set(x_91, 0, x_90); +lean_closure_set(x_91, 1, x_89); +x_92 = l_Task_Priority_default; +x_93 = lean_io_as_task(x_91, x_92, x_13); +if (lean_obj_tag(x_93) == 0) +{ +uint8_t x_94; +x_94 = !lean_is_exclusive(x_93); +if (x_94 == 0) +{ +lean_object* x_95; lean_object* x_96; +x_95 = lean_ctor_get(x_93, 0); +lean_dec(x_95); +x_96 = lean_box(0); +lean_ctor_set(x_93, 0, x_96); +return x_93; +} +else +{ +lean_object* x_97; lean_object* x_98; lean_object* x_99; +x_97 = lean_ctor_get(x_93, 1); +lean_inc(x_97); +lean_dec(x_93); +x_98 = lean_box(0); +x_99 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_99, 0, x_98); +lean_ctor_set(x_99, 1, x_97); +return x_99; +} +} +else +{ +uint8_t x_100; +x_100 = !lean_is_exclusive(x_93); +if (x_100 == 0) +{ +return x_93; +} +else +{ +lean_object* x_101; lean_object* x_102; lean_object* x_103; +x_101 = lean_ctor_get(x_93, 0); +x_102 = lean_ctor_get(x_93, 1); +lean_inc(x_102); +lean_inc(x_101); +lean_dec(x_93); +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; +} +} +} +} +} +static lean_object* _init_l_Lean_Language_Lean_process_parseCmd___lambda__5___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; +x_1 = lean_box(0); +x_2 = l_Lean_Language_Lean_process_parseCmd___lambda__2___closed__3; +x_3 = l_Lean_Language_Snapshot_Diagnostics_empty; +x_4 = 0; +x_5 = lean_alloc_ctor(0, 3, 1); +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_uint8(x_5, sizeof(void*)*3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Language_Lean_process_parseCmd___lambda__5___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Language_instTypeNameSnapshotLeaf; +x_2 = l_Lean_Language_Lean_process_parseCmd___lambda__5___closed__1; +x_3 = l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Language_instInhabitedDynamicSnapshot___spec__1(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Language_Lean_process_parseCmd___lambda__5___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Language_Lean_process_parseCmd___lambda__5___closed__2; +x_2 = l_Lean_Language_SnapshotTask_pure___rarg(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__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, 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; +x_14 = lean_ctor_get(x_1, 3); +lean_inc(x_14); +x_15 = lean_st_ref_get(x_14, x_13); +lean_dec(x_14); +if (lean_obj_tag(x_15) == 0) +{ +lean_object* x_16; uint8_t x_17; +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +x_17 = lean_unbox(x_16); +lean_dec(x_16); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_15, 1); +lean_inc(x_18); +lean_dec(x_15); +x_19 = lean_box(0); +x_20 = l_Lean_Language_Lean_process_parseCmd___lambda__4(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_1, x_10, x_19, x_12, x_18); +return x_20; +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; +lean_dec(x_9); +lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_21 = lean_ctor_get(x_15, 1); +lean_inc(x_21); +lean_dec(x_15); +x_22 = l_Lean_Language_Lean_process_parseCmd___lambda__3___closed__1; +x_23 = lean_st_mk_ref(x_22, x_21); +if (lean_obj_tag(x_23) == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +x_26 = lean_box(0); +x_27 = l_Lean_Language_Lean_process_parseCmd___lambda__5___closed__1; +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_8); +x_29 = l_Lean_Language_SnapshotTask_pure___rarg(x_28); +x_30 = lean_box(0); +x_31 = l_Lean_Language_Lean_process_parseCmd___lambda__5___closed__3; +x_32 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_32, 0, x_27); +lean_ctor_set(x_32, 1, x_30); +lean_ctor_set(x_32, 2, x_10); +lean_ctor_set(x_32, 3, x_31); +lean_ctor_set(x_32, 4, x_29); +lean_ctor_set(x_32, 5, x_24); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_26); +x_34 = lean_io_promise_resolve(x_33, x_6, x_25); +lean_dec(x_6); +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; lean_object* x_37; +x_36 = lean_ctor_get(x_34, 0); +lean_dec(x_36); +x_37 = lean_box(0); +lean_ctor_set(x_34, 0, x_37); +return x_34; +} +else +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_34, 1); +lean_inc(x_38); +lean_dec(x_34); +x_39 = lean_box(0); +x_40 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_40, 0, x_39); +lean_ctor_set(x_40, 1, x_38); +return x_40; +} +} +else +{ +uint8_t x_41; +x_41 = !lean_is_exclusive(x_34); +if (x_41 == 0) +{ +return x_34; +} +else +{ +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 +{ +uint8_t x_45; +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_6); +x_45 = !lean_is_exclusive(x_23); +if (x_45 == 0) +{ +return x_23; +} +else +{ +lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_46 = lean_ctor_get(x_23, 0); +x_47 = lean_ctor_get(x_23, 1); +lean_inc(x_47); +lean_inc(x_46); +lean_dec(x_23); +x_48 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_48, 0, x_46); +lean_ctor_set(x_48, 1, x_47); +return x_48; +} +} +} +} +else +{ +uint8_t x_49; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_49 = !lean_is_exclusive(x_15); +if (x_49 == 0) +{ +return x_15; +} +else +{ +lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_50 = lean_ctor_get(x_15, 0); +x_51 = lean_ctor_get(x_15, 1); +lean_inc(x_51); +lean_inc(x_50); +lean_dec(x_15); +x_52 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_52, 0, x_50); +lean_ctor_set(x_52, 1, x_51); +return x_52; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___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; +x_6 = lean_ctor_get(x_1, 2); +if (lean_obj_tag(x_6) == 0) +{ +lean_object* x_7; lean_object* x_8; +x_7 = lean_box(0); +x_8 = lean_apply_3(x_2, x_7, x_4, x_5); +return x_8; +} +else +{ +lean_object* x_9; uint8_t x_10; lean_object* x_11; lean_object* x_12; +x_9 = lean_ctor_get(x_6, 0); +x_10 = 1; +x_11 = lean_box(x_10); +x_12 = lean_st_ref_set(x_9, x_11, x_5); +if (lean_obj_tag(x_12) == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_12, 1); +lean_inc(x_14); +lean_dec(x_12); +x_15 = lean_apply_3(x_2, x_13, x_4, x_14); +return x_15; +} +else +{ +uint8_t x_16; +lean_dec(x_4); +lean_dec(x_2); +x_16 = !lean_is_exclusive(x_12); +if (x_16 == 0) +{ +return x_12; +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_12, 0); +x_18 = lean_ctor_get(x_12, 1); +lean_inc(x_18); +lean_inc(x_17); +lean_dec(x_12); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set(x_19, 1, x_18); +return x_19; +} +} +} +} +} +static lean_object* _init_l_Lean_Language_Lean_process_parseCmd___lambda__7___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = l_Lean_Language_SnapshotTask_pure___rarg(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_6); +x_9 = lean_ctor_get(x_1, 1); +lean_inc(x_9); +lean_dec(x_1); +x_10 = l_Lean_Language_Lean_process_parseCmd(x_8, x_2, x_9, x_3, x_4, x_5, x_7); +if (lean_obj_tag(x_10) == 0) +{ +uint8_t x_11; +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; +x_12 = lean_ctor_get(x_10, 0); +lean_dec(x_12); +x_13 = l_Lean_Language_Lean_process_parseCmd___lambda__7___closed__1; +lean_ctor_set(x_10, 0, x_13); +return x_10; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_10, 1); +lean_inc(x_14); +lean_dec(x_10); +x_15 = l_Lean_Language_Lean_process_parseCmd___lambda__7___closed__1; +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_16, 1, x_14); +return x_16; +} +} +else +{ +uint8_t x_17; +x_17 = !lean_is_exclusive(x_10); +if (x_17 == 0) +{ +return x_10; +} +else +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_10, 0); +x_19 = lean_ctor_get(x_10, 1); +lean_inc(x_19); +lean_inc(x_18); +lean_dec(x_10); +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_Language_Lean_process_parseCmd___lambda__8(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; lean_object* x_12; +x_8 = lean_box(x_3); +x_9 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_parseCmd___lambda__7___boxed), 7, 5); +lean_closure_set(x_9, 0, x_6); +lean_closure_set(x_9, 1, x_1); +lean_closure_set(x_9, 2, x_2); +lean_closure_set(x_9, 3, x_8); +lean_closure_set(x_9, 4, x_4); +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +x_11 = 1; +x_12 = l_Lean_Language_SnapshotTask_bindIO___rarg(x_5, x_9, x_10, x_11, x_7); +return x_12; +} +} +static lean_object* _init_l_Lean_Language_Lean_process_parseCmd___lambda__9___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("parsing", 7, 7); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; 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_ctor_get(x_1, 0); +lean_inc(x_10); +x_11 = lean_ctor_get(x_2, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_2, 2); +lean_inc(x_12); +x_13 = l_Lean_Elab_Command_instInhabitedScope; +x_14 = l_List_head_x21___rarg(x_13, x_12); +lean_dec(x_12); +x_15 = lean_ctor_get(x_14, 1); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 2); +lean_inc(x_16); +x_17 = lean_ctor_get(x_14, 3); +lean_inc(x_17); +lean_dec(x_14); +lean_inc(x_15); +x_18 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_18, 0, x_11); +lean_ctor_set(x_18, 1, x_15); +lean_ctor_set(x_18, 2, x_16); +lean_ctor_set(x_18, 3, x_17); +lean_inc(x_3); +x_19 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_parseCmd___lambda__1___boxed), 4, 3); +lean_closure_set(x_19, 0, x_3); +lean_closure_set(x_19, 1, x_18); +lean_closure_set(x_19, 2, x_1); +x_20 = l_Lean_Language_Lean_process_parseCmd___lambda__9___closed__1; +x_21 = lean_box(0); +x_22 = lean_profileit(x_20, x_15, x_19, x_21); +x_23 = lean_ctor_get(x_22, 1); +lean_inc(x_23); +if (lean_obj_tag(x_6) == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_24 = lean_ctor_get(x_22, 0); +lean_inc(x_24); +lean_dec(x_22); +x_25 = lean_ctor_get(x_23, 0); +lean_inc(x_25); +x_26 = lean_ctor_get(x_23, 1); +lean_inc(x_26); +lean_dec(x_23); +x_27 = lean_box(0); +x_28 = l_Lean_Language_Lean_process_parseCmd___lambda__5(x_3, x_4, x_24, x_15, x_26, x_5, x_6, x_2, x_10, x_25, x_27, x_8, x_9); +lean_dec(x_8); +return x_28; +} +else +{ +lean_object* x_29; uint8_t x_30; +x_29 = lean_ctor_get(x_22, 0); +lean_inc(x_29); +lean_dec(x_22); +x_30 = !lean_is_exclusive(x_23); +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; uint8_t x_39; +x_31 = lean_ctor_get(x_23, 0); +x_32 = lean_ctor_get(x_23, 1); +x_33 = lean_ctor_get(x_6, 0); +lean_inc(x_33); +x_34 = lean_box(x_4); +lean_inc(x_31); +lean_inc(x_5); +lean_inc(x_29); +lean_inc(x_3); +x_35 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_parseCmd___lambda__5___boxed), 13, 10); +lean_closure_set(x_35, 0, x_3); +lean_closure_set(x_35, 1, x_34); +lean_closure_set(x_35, 2, x_29); +lean_closure_set(x_35, 3, x_15); +lean_closure_set(x_35, 4, x_32); +lean_closure_set(x_35, 5, x_5); +lean_closure_set(x_35, 6, x_6); +lean_closure_set(x_35, 7, x_2); +lean_closure_set(x_35, 8, x_10); +lean_closure_set(x_35, 9, x_31); +x_36 = lean_ctor_get(x_33, 0); +lean_inc(x_36); +x_37 = lean_ctor_get(x_33, 1); +lean_inc(x_37); +x_38 = lean_ctor_get(x_36, 1); +lean_inc(x_38); +x_39 = l_Lean_Syntax_eqWithInfo(x_29, x_38); +if (x_39 == 0) +{ +lean_object* x_40; lean_object* x_41; +lean_dec(x_37); +lean_dec(x_36); +lean_dec(x_33); +lean_free_object(x_23); +lean_dec(x_31); +lean_dec(x_5); +x_40 = lean_box(0); +x_41 = l_Lean_Language_Lean_process_parseCmd___lambda__6(x_3, x_35, x_40, x_8, x_9); +lean_dec(x_3); +return x_41; +} +else +{ +lean_dec(x_35); +lean_dec(x_8); +if (lean_obj_tag(x_37) == 0) +{ +lean_object* x_42; +lean_dec(x_36); +lean_free_object(x_23); +lean_dec(x_31); +lean_dec(x_3); +x_42 = lean_io_promise_resolve(x_33, x_5, x_9); +lean_dec(x_5); +if (lean_obj_tag(x_42) == 0) +{ +uint8_t x_43; +x_43 = !lean_is_exclusive(x_42); +if (x_43 == 0) +{ +return x_42; +} +else +{ +lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_44 = lean_ctor_get(x_42, 0); +x_45 = lean_ctor_get(x_42, 1); +lean_inc(x_45); +lean_inc(x_44); +lean_dec(x_42); +x_46 = lean_alloc_ctor(0, 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; +x_47 = !lean_is_exclusive(x_42); +if (x_47 == 0) +{ +return x_42; +} +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; +} +} +} +else +{ +uint8_t x_51; +x_51 = !lean_is_exclusive(x_33); +if (x_51 == 0) +{ +lean_object* x_52; lean_object* x_53; uint8_t x_54; +x_52 = lean_ctor_get(x_33, 1); +lean_dec(x_52); +x_53 = lean_ctor_get(x_33, 0); +lean_dec(x_53); +x_54 = !lean_is_exclusive(x_37); +if (x_54 == 0) +{ +lean_object* x_55; lean_object* x_56; +x_55 = lean_ctor_get(x_37, 0); +x_56 = lean_io_promise_new(x_9); +if (lean_obj_tag(x_56) == 0) +{ +lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; lean_object* x_64; +x_57 = lean_ctor_get(x_56, 0); +lean_inc(x_57); +x_58 = lean_ctor_get(x_56, 1); +lean_inc(x_58); +lean_dec(x_56); +x_59 = lean_box(x_4); +lean_inc(x_57); +x_60 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_parseCmd___lambda__8___boxed), 7, 5); +lean_closure_set(x_60, 0, x_31); +lean_closure_set(x_60, 1, x_57); +lean_closure_set(x_60, 2, x_59); +lean_closure_set(x_60, 3, x_3); +lean_closure_set(x_60, 4, x_55); +x_61 = lean_ctor_get(x_36, 4); +lean_inc(x_61); +x_62 = lean_ctor_get(x_61, 0); +lean_inc(x_62); +x_63 = 1; +x_64 = l_Lean_Language_SnapshotTask_bindIO___rarg(x_61, x_60, x_62, x_63, x_58); +if (lean_obj_tag(x_64) == 0) +{ +lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; +x_65 = lean_ctor_get(x_64, 1); +lean_inc(x_65); +lean_dec(x_64); +x_66 = lean_box(0); +x_67 = lean_io_promise_result(x_57); +lean_ctor_set(x_23, 1, x_67); +lean_ctor_set(x_23, 0, x_66); +lean_ctor_set(x_37, 0, x_23); +x_68 = lean_io_promise_resolve(x_33, x_5, x_65); +lean_dec(x_5); +if (lean_obj_tag(x_68) == 0) +{ +uint8_t x_69; +x_69 = !lean_is_exclusive(x_68); +if (x_69 == 0) +{ +return x_68; } +else +{ +lean_object* x_70; lean_object* x_71; lean_object* x_72; +x_70 = lean_ctor_get(x_68, 0); +x_71 = lean_ctor_get(x_68, 1); +lean_inc(x_71); +lean_inc(x_70); +lean_dec(x_68); +x_72 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_72, 0, x_70); +lean_ctor_set(x_72, 1, x_71); +return x_72; } } else { -uint8_t x_78; -lean_free_object(x_35); -lean_dec(x_53); -lean_free_object(x_32); -lean_dec(x_34); -lean_free_object(x_22); -lean_dec(x_30); -lean_dec(x_4); -lean_dec(x_3); -x_78 = !lean_is_exclusive(x_54); -if (x_78 == 0) +uint8_t x_73; +x_73 = !lean_is_exclusive(x_68); +if (x_73 == 0) { -return x_54; +return x_68; } else { -lean_object* x_79; lean_object* x_80; lean_object* x_81; -x_79 = lean_ctor_get(x_54, 0); -x_80 = lean_ctor_get(x_54, 1); -lean_inc(x_80); +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; +} +} +} +else +{ +uint8_t x_77; +lean_dec(x_57); +lean_free_object(x_37); +lean_free_object(x_33); +lean_dec(x_36); +lean_free_object(x_23); +lean_dec(x_5); +x_77 = !lean_is_exclusive(x_64); +if (x_77 == 0) +{ +return x_64; +} +else +{ +lean_object* x_78; lean_object* x_79; lean_object* x_80; +x_78 = lean_ctor_get(x_64, 0); +x_79 = lean_ctor_get(x_64, 1); lean_inc(x_79); -lean_dec(x_54); -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_inc(x_78); +lean_dec(x_64); +x_80 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_80, 0, x_78); +lean_ctor_set(x_80, 1, x_79); +return x_80; } } } else { -lean_object* x_82; lean_object* x_83; -x_82 = lean_ctor_get(x_35, 0); +uint8_t x_81; +lean_free_object(x_37); +lean_dec(x_55); +lean_free_object(x_33); +lean_dec(x_36); +lean_free_object(x_23); +lean_dec(x_31); +lean_dec(x_5); +lean_dec(x_3); +x_81 = !lean_is_exclusive(x_56); +if (x_81 == 0) +{ +return x_56; +} +else +{ +lean_object* x_82; lean_object* x_83; lean_object* x_84; +x_82 = lean_ctor_get(x_56, 0); +x_83 = lean_ctor_get(x_56, 1); +lean_inc(x_83); lean_inc(x_82); -lean_dec(x_35); -x_83 = lean_io_promise_new(x_8); -if (lean_obj_tag(x_83) == 0) +lean_dec(x_56); +x_84 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_84, 0, x_82); +lean_ctor_set(x_84, 1, x_83); +return x_84; +} +} +} +else { -lean_object* x_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_84 = lean_ctor_get(x_83, 0); -lean_inc(x_84); -x_85 = lean_ctor_get(x_83, 1); +lean_object* x_85; lean_object* x_86; +x_85 = lean_ctor_get(x_37, 0); lean_inc(x_85); -lean_dec(x_83); -lean_inc(x_84); -x_86 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_parseCmd___lambda__6), 6, 4); -lean_closure_set(x_86, 0, x_30); -lean_closure_set(x_86, 1, x_84); -lean_closure_set(x_86, 2, x_3); -lean_closure_set(x_86, 3, x_82); -x_87 = lean_ctor_get(x_34, 4); +lean_dec(x_37); +x_86 = lean_io_promise_new(x_9); +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; uint8_t x_93; lean_object* x_94; +x_87 = lean_ctor_get(x_86, 0); lean_inc(x_87); -x_88 = lean_ctor_get(x_87, 0); +x_88 = lean_ctor_get(x_86, 1); lean_inc(x_88); -x_89 = 0; -x_90 = l_Lean_Language_SnapshotTask_bindIO___rarg(x_87, x_86, x_88, x_89, x_85); -if (lean_obj_tag(x_90) == 0) -{ -lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; -x_91 = lean_ctor_get(x_90, 1); +lean_dec(x_86); +x_89 = lean_box(x_4); +lean_inc(x_87); +x_90 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_parseCmd___lambda__8___boxed), 7, 5); +lean_closure_set(x_90, 0, x_31); +lean_closure_set(x_90, 1, x_87); +lean_closure_set(x_90, 2, x_89); +lean_closure_set(x_90, 3, x_3); +lean_closure_set(x_90, 4, x_85); +x_91 = lean_ctor_get(x_36, 4); lean_inc(x_91); -lean_dec(x_90); -x_92 = lean_box(0); -x_93 = lean_io_promise_result(x_84); -lean_ctor_set(x_22, 1, x_93); -lean_ctor_set(x_22, 0, x_92); -x_94 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_94, 0, x_22); -lean_ctor_set(x_32, 1, x_94); -x_95 = lean_io_promise_resolve(x_32, x_4, x_91); -lean_dec(x_4); -if (lean_obj_tag(x_95) == 0) +x_92 = lean_ctor_get(x_91, 0); +lean_inc(x_92); +x_93 = 1; +x_94 = l_Lean_Language_SnapshotTask_bindIO___rarg(x_91, x_90, x_92, x_93, x_88); +if (lean_obj_tag(x_94) == 0) { -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); -if (lean_is_exclusive(x_95)) { - lean_ctor_release(x_95, 0); - lean_ctor_release(x_95, 1); - x_98 = x_95; -} else { - lean_dec_ref(x_95); - x_98 = lean_box(0); -} -if (lean_is_scalar(x_98)) { - x_99 = lean_alloc_ctor(0, 2, 0); -} else { - x_99 = x_98; -} -lean_ctor_set(x_99, 0, x_96); -lean_ctor_set(x_99, 1, x_97); -return x_99; -} -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_94, 1); +lean_inc(x_95); +lean_dec(x_94); +x_96 = lean_box(0); +x_97 = lean_io_promise_result(x_87); +lean_ctor_set(x_23, 1, x_97); +lean_ctor_set(x_23, 0, x_96); +x_98 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_98, 0, x_23); +lean_ctor_set(x_33, 1, x_98); +x_99 = lean_io_promise_resolve(x_33, x_5, x_95); +lean_dec(x_5); +if (lean_obj_tag(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_95, 0); +x_100 = lean_ctor_get(x_99, 0); lean_inc(x_100); -x_101 = lean_ctor_get(x_95, 1); +x_101 = lean_ctor_get(x_99, 1); lean_inc(x_101); -if (lean_is_exclusive(x_95)) { - lean_ctor_release(x_95, 0); - lean_ctor_release(x_95, 1); - x_102 = x_95; +if (lean_is_exclusive(x_99)) { + lean_ctor_release(x_99, 0); + lean_ctor_release(x_99, 1); + x_102 = x_99; } else { - lean_dec_ref(x_95); + lean_dec_ref(x_99); x_102 = lean_box(0); } if (lean_is_scalar(x_102)) { - x_103 = lean_alloc_ctor(1, 2, 0); + x_103 = lean_alloc_ctor(0, 2, 0); } else { x_103 = x_102; } @@ -6024,25 +6640,19 @@ lean_ctor_set(x_103, 0, x_100); lean_ctor_set(x_103, 1, x_101); return x_103; } -} else { lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; -lean_dec(x_84); -lean_free_object(x_32); -lean_dec(x_34); -lean_free_object(x_22); -lean_dec(x_4); -x_104 = lean_ctor_get(x_90, 0); +x_104 = lean_ctor_get(x_99, 0); lean_inc(x_104); -x_105 = lean_ctor_get(x_90, 1); +x_105 = lean_ctor_get(x_99, 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; +if (lean_is_exclusive(x_99)) { + lean_ctor_release(x_99, 0); + lean_ctor_release(x_99, 1); + x_106 = x_99; } else { - lean_dec_ref(x_90); + lean_dec_ref(x_99); x_106 = lean_box(0); } if (lean_is_scalar(x_106)) { @@ -6058,23 +6668,21 @@ return x_107; else { lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; -lean_dec(x_82); -lean_free_object(x_32); -lean_dec(x_34); -lean_free_object(x_22); -lean_dec(x_30); -lean_dec(x_4); -lean_dec(x_3); -x_108 = lean_ctor_get(x_83, 0); +lean_dec(x_87); +lean_free_object(x_33); +lean_dec(x_36); +lean_free_object(x_23); +lean_dec(x_5); +x_108 = lean_ctor_get(x_94, 0); lean_inc(x_108); -x_109 = lean_ctor_get(x_83, 1); +x_109 = lean_ctor_get(x_94, 1); lean_inc(x_109); -if (lean_is_exclusive(x_83)) { - lean_ctor_release(x_83, 0); - lean_ctor_release(x_83, 1); - x_110 = x_83; +if (lean_is_exclusive(x_94)) { + lean_ctor_release(x_94, 0); + lean_ctor_release(x_94, 1); + x_110 = x_94; } else { - lean_dec_ref(x_83); + lean_dec_ref(x_94); x_110 = lean_box(0); } if (lean_is_scalar(x_110)) { @@ -6087,171 +6695,205 @@ lean_ctor_set(x_111, 1, x_109); return x_111; } } -} else { -lean_object* x_112; lean_object* x_113; lean_object* x_114; -lean_dec(x_32); -x_112 = lean_ctor_get(x_35, 0); +lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; +lean_dec(x_85); +lean_free_object(x_33); +lean_dec(x_36); +lean_free_object(x_23); +lean_dec(x_31); +lean_dec(x_5); +lean_dec(x_3); +x_112 = lean_ctor_get(x_86, 0); lean_inc(x_112); -if (lean_is_exclusive(x_35)) { - lean_ctor_release(x_35, 0); - x_113 = x_35; +x_113 = lean_ctor_get(x_86, 1); +lean_inc(x_113); +if (lean_is_exclusive(x_86)) { + lean_ctor_release(x_86, 0); + lean_ctor_release(x_86, 1); + x_114 = x_86; +} else { + lean_dec_ref(x_86); + x_114 = lean_box(0); +} +if (lean_is_scalar(x_114)) { + x_115 = lean_alloc_ctor(1, 2, 0); } else { - lean_dec_ref(x_35); - x_113 = lean_box(0); + x_115 = x_114; +} +lean_ctor_set(x_115, 0, x_112); +lean_ctor_set(x_115, 1, x_113); +return x_115; } -x_114 = lean_io_promise_new(x_8); -if (lean_obj_tag(x_114) == 0) +} +} +else { -lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; uint8_t x_120; lean_object* x_121; -x_115 = lean_ctor_get(x_114, 0); -lean_inc(x_115); -x_116 = lean_ctor_get(x_114, 1); +lean_object* x_116; lean_object* x_117; lean_object* x_118; +lean_dec(x_33); +x_116 = lean_ctor_get(x_37, 0); lean_inc(x_116); -lean_dec(x_114); -lean_inc(x_115); -x_117 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_parseCmd___lambda__6), 6, 4); -lean_closure_set(x_117, 0, x_30); -lean_closure_set(x_117, 1, x_115); -lean_closure_set(x_117, 2, x_3); -lean_closure_set(x_117, 3, x_112); -x_118 = lean_ctor_get(x_34, 4); -lean_inc(x_118); +if (lean_is_exclusive(x_37)) { + lean_ctor_release(x_37, 0); + x_117 = x_37; +} else { + lean_dec_ref(x_37); + x_117 = lean_box(0); +} +x_118 = lean_io_promise_new(x_9); +if (lean_obj_tag(x_118) == 0) +{ +lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; uint8_t x_125; lean_object* x_126; x_119 = lean_ctor_get(x_118, 0); lean_inc(x_119); -x_120 = 0; -x_121 = l_Lean_Language_SnapshotTask_bindIO___rarg(x_118, x_117, x_119, x_120, x_116); -if (lean_obj_tag(x_121) == 0) +x_120 = lean_ctor_get(x_118, 1); +lean_inc(x_120); +lean_dec(x_118); +x_121 = lean_box(x_4); +lean_inc(x_119); +x_122 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_parseCmd___lambda__8___boxed), 7, 5); +lean_closure_set(x_122, 0, x_31); +lean_closure_set(x_122, 1, x_119); +lean_closure_set(x_122, 2, x_121); +lean_closure_set(x_122, 3, x_3); +lean_closure_set(x_122, 4, x_116); +x_123 = lean_ctor_get(x_36, 4); +lean_inc(x_123); +x_124 = lean_ctor_get(x_123, 0); +lean_inc(x_124); +x_125 = 1; +x_126 = l_Lean_Language_SnapshotTask_bindIO___rarg(x_123, x_122, x_124, x_125, x_120); +if (lean_obj_tag(x_126) == 0) { -lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; -x_122 = lean_ctor_get(x_121, 1); -lean_inc(x_122); -lean_dec(x_121); -x_123 = lean_box(0); -x_124 = lean_io_promise_result(x_115); -lean_ctor_set(x_22, 1, x_124); -lean_ctor_set(x_22, 0, x_123); -if (lean_is_scalar(x_113)) { - x_125 = lean_alloc_ctor(1, 1, 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; +x_127 = lean_ctor_get(x_126, 1); +lean_inc(x_127); +lean_dec(x_126); +x_128 = lean_box(0); +x_129 = lean_io_promise_result(x_119); +lean_ctor_set(x_23, 1, x_129); +lean_ctor_set(x_23, 0, x_128); +if (lean_is_scalar(x_117)) { + x_130 = lean_alloc_ctor(1, 1, 0); } else { - x_125 = x_113; + x_130 = x_117; } -lean_ctor_set(x_125, 0, x_22); -x_126 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_126, 0, x_34); -lean_ctor_set(x_126, 1, x_125); -x_127 = lean_io_promise_resolve(x_126, x_4, x_122); -lean_dec(x_4); -if (lean_obj_tag(x_127) == 0) +lean_ctor_set(x_130, 0, x_23); +x_131 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_131, 0, x_36); +lean_ctor_set(x_131, 1, x_130); +x_132 = lean_io_promise_resolve(x_131, x_5, x_127); +lean_dec(x_5); +if (lean_obj_tag(x_132) == 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); -if (lean_is_exclusive(x_127)) { - lean_ctor_release(x_127, 0); - lean_ctor_release(x_127, 1); - x_130 = x_127; +lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; +x_133 = lean_ctor_get(x_132, 0); +lean_inc(x_133); +x_134 = lean_ctor_get(x_132, 1); +lean_inc(x_134); +if (lean_is_exclusive(x_132)) { + lean_ctor_release(x_132, 0); + lean_ctor_release(x_132, 1); + x_135 = x_132; } else { - lean_dec_ref(x_127); - x_130 = lean_box(0); + lean_dec_ref(x_132); + x_135 = lean_box(0); } -if (lean_is_scalar(x_130)) { - x_131 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_135)) { + x_136 = lean_alloc_ctor(0, 2, 0); } else { - x_131 = x_130; + x_136 = x_135; } -lean_ctor_set(x_131, 0, x_128); -lean_ctor_set(x_131, 1, x_129); -return x_131; +lean_ctor_set(x_136, 0, x_133); +lean_ctor_set(x_136, 1, x_134); +return x_136; } else { -lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; -x_132 = lean_ctor_get(x_127, 0); -lean_inc(x_132); -x_133 = lean_ctor_get(x_127, 1); -lean_inc(x_133); -if (lean_is_exclusive(x_127)) { - lean_ctor_release(x_127, 0); - lean_ctor_release(x_127, 1); - x_134 = x_127; +lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; +x_137 = lean_ctor_get(x_132, 0); +lean_inc(x_137); +x_138 = lean_ctor_get(x_132, 1); +lean_inc(x_138); +if (lean_is_exclusive(x_132)) { + lean_ctor_release(x_132, 0); + lean_ctor_release(x_132, 1); + x_139 = x_132; } else { - lean_dec_ref(x_127); - x_134 = lean_box(0); + lean_dec_ref(x_132); + x_139 = lean_box(0); } -if (lean_is_scalar(x_134)) { - x_135 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_139)) { + x_140 = lean_alloc_ctor(1, 2, 0); } else { - x_135 = x_134; + x_140 = x_139; } -lean_ctor_set(x_135, 0, x_132); -lean_ctor_set(x_135, 1, x_133); -return x_135; +lean_ctor_set(x_140, 0, x_137); +lean_ctor_set(x_140, 1, x_138); +return x_140; } } else { -lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; -lean_dec(x_115); -lean_dec(x_113); -lean_dec(x_34); -lean_free_object(x_22); -lean_dec(x_4); -x_136 = lean_ctor_get(x_121, 0); -lean_inc(x_136); -x_137 = lean_ctor_get(x_121, 1); -lean_inc(x_137); -if (lean_is_exclusive(x_121)) { - lean_ctor_release(x_121, 0); - lean_ctor_release(x_121, 1); - x_138 = x_121; +lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; +lean_dec(x_119); +lean_dec(x_117); +lean_dec(x_36); +lean_free_object(x_23); +lean_dec(x_5); +x_141 = lean_ctor_get(x_126, 0); +lean_inc(x_141); +x_142 = lean_ctor_get(x_126, 1); +lean_inc(x_142); +if (lean_is_exclusive(x_126)) { + lean_ctor_release(x_126, 0); + lean_ctor_release(x_126, 1); + x_143 = x_126; } else { - lean_dec_ref(x_121); - x_138 = lean_box(0); + lean_dec_ref(x_126); + x_143 = lean_box(0); } -if (lean_is_scalar(x_138)) { - x_139 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_143)) { + x_144 = lean_alloc_ctor(1, 2, 0); } else { - x_139 = x_138; + x_144 = x_143; } -lean_ctor_set(x_139, 0, x_136); -lean_ctor_set(x_139, 1, x_137); -return x_139; +lean_ctor_set(x_144, 0, x_141); +lean_ctor_set(x_144, 1, x_142); +return x_144; } } else { -lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; -lean_dec(x_113); -lean_dec(x_112); -lean_dec(x_34); -lean_free_object(x_22); -lean_dec(x_30); -lean_dec(x_4); +lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; +lean_dec(x_117); +lean_dec(x_116); +lean_dec(x_36); +lean_free_object(x_23); +lean_dec(x_31); +lean_dec(x_5); lean_dec(x_3); -x_140 = lean_ctor_get(x_114, 0); -lean_inc(x_140); -x_141 = lean_ctor_get(x_114, 1); -lean_inc(x_141); -if (lean_is_exclusive(x_114)) { - lean_ctor_release(x_114, 0); - lean_ctor_release(x_114, 1); - x_142 = x_114; +x_145 = lean_ctor_get(x_118, 0); +lean_inc(x_145); +x_146 = lean_ctor_get(x_118, 1); +lean_inc(x_146); +if (lean_is_exclusive(x_118)) { + lean_ctor_release(x_118, 0); + lean_ctor_release(x_118, 1); + x_147 = x_118; } else { - lean_dec_ref(x_114); - x_142 = lean_box(0); + lean_dec_ref(x_118); + x_147 = lean_box(0); } -if (lean_is_scalar(x_142)) { - x_143 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_147)) { + x_148 = lean_alloc_ctor(1, 2, 0); } else { - x_143 = x_142; + x_148 = x_147; } -lean_ctor_set(x_143, 0, x_140); -lean_ctor_set(x_143, 1, x_141); -return x_143; +lean_ctor_set(x_148, 0, x_145); +lean_ctor_set(x_148, 1, x_146); +return x_148; } } } @@ -6259,285 +6901,289 @@ return x_143; } else { -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; uint8_t x_151; -x_144 = lean_ctor_get(x_22, 0); -x_145 = lean_ctor_get(x_22, 1); -lean_inc(x_145); -lean_inc(x_144); -lean_dec(x_22); -x_146 = lean_ctor_get(x_5, 0); -lean_inc(x_146); -lean_inc(x_144); -lean_inc(x_3); -lean_inc(x_4); -lean_inc(x_28); -x_147 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_parseCmd___lambda__3___boxed), 12, 9); -lean_closure_set(x_147, 0, x_28); -lean_closure_set(x_147, 1, x_14); -lean_closure_set(x_147, 2, x_145); -lean_closure_set(x_147, 3, x_4); -lean_closure_set(x_147, 4, x_5); -lean_closure_set(x_147, 5, x_2); -lean_closure_set(x_147, 6, x_9); -lean_closure_set(x_147, 7, x_3); -lean_closure_set(x_147, 8, x_144); -x_148 = lean_ctor_get(x_146, 0); -lean_inc(x_148); -x_149 = lean_ctor_get(x_146, 1); -lean_inc(x_149); -x_150 = lean_ctor_get(x_148, 1); +lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; uint8_t x_157; +x_149 = lean_ctor_get(x_23, 0); +x_150 = lean_ctor_get(x_23, 1); lean_inc(x_150); -x_151 = l_Lean_Syntax_eqWithInfo(x_28, x_150); -if (x_151 == 0) +lean_inc(x_149); +lean_dec(x_23); +x_151 = lean_ctor_get(x_6, 0); +lean_inc(x_151); +x_152 = lean_box(x_4); +lean_inc(x_149); +lean_inc(x_5); +lean_inc(x_29); +lean_inc(x_3); +x_153 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_parseCmd___lambda__5___boxed), 13, 10); +lean_closure_set(x_153, 0, x_3); +lean_closure_set(x_153, 1, x_152); +lean_closure_set(x_153, 2, x_29); +lean_closure_set(x_153, 3, x_15); +lean_closure_set(x_153, 4, x_150); +lean_closure_set(x_153, 5, x_5); +lean_closure_set(x_153, 6, x_6); +lean_closure_set(x_153, 7, x_2); +lean_closure_set(x_153, 8, x_10); +lean_closure_set(x_153, 9, x_149); +x_154 = lean_ctor_get(x_151, 0); +lean_inc(x_154); +x_155 = lean_ctor_get(x_151, 1); +lean_inc(x_155); +x_156 = lean_ctor_get(x_154, 1); +lean_inc(x_156); +x_157 = l_Lean_Syntax_eqWithInfo(x_29, x_156); +if (x_157 == 0) { -lean_object* x_152; lean_object* x_153; +lean_object* x_158; lean_object* x_159; +lean_dec(x_155); +lean_dec(x_154); +lean_dec(x_151); lean_dec(x_149); -lean_dec(x_148); -lean_dec(x_146); -lean_dec(x_144); -lean_dec(x_4); -x_152 = lean_box(0); -x_153 = l_Lean_Language_Lean_process_parseCmd___lambda__4(x_3, x_147, x_152, x_7, x_8); +lean_dec(x_5); +x_158 = lean_box(0); +x_159 = l_Lean_Language_Lean_process_parseCmd___lambda__6(x_3, x_153, x_158, x_8, x_9); lean_dec(x_3); -return x_153; +return x_159; } else { -lean_dec(x_147); -lean_dec(x_7); -if (lean_obj_tag(x_149) == 0) +lean_dec(x_153); +lean_dec(x_8); +if (lean_obj_tag(x_155) == 0) { -lean_object* x_154; -lean_dec(x_148); -lean_dec(x_144); +lean_object* x_160; +lean_dec(x_154); +lean_dec(x_149); lean_dec(x_3); -x_154 = lean_io_promise_resolve(x_146, x_4, x_8); -lean_dec(x_4); -if (lean_obj_tag(x_154) == 0) +x_160 = lean_io_promise_resolve(x_151, x_5, x_9); +lean_dec(x_5); +if (lean_obj_tag(x_160) == 0) { -lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; -x_155 = lean_ctor_get(x_154, 0); -lean_inc(x_155); -x_156 = lean_ctor_get(x_154, 1); -lean_inc(x_156); -if (lean_is_exclusive(x_154)) { - lean_ctor_release(x_154, 0); - lean_ctor_release(x_154, 1); - x_157 = x_154; +lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; +x_161 = lean_ctor_get(x_160, 0); +lean_inc(x_161); +x_162 = lean_ctor_get(x_160, 1); +lean_inc(x_162); +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_154); - x_157 = lean_box(0); + lean_dec_ref(x_160); + x_163 = lean_box(0); } -if (lean_is_scalar(x_157)) { - x_158 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_163)) { + x_164 = lean_alloc_ctor(0, 2, 0); } else { - x_158 = x_157; + x_164 = x_163; } -lean_ctor_set(x_158, 0, x_155); -lean_ctor_set(x_158, 1, x_156); -return x_158; +lean_ctor_set(x_164, 0, x_161); +lean_ctor_set(x_164, 1, x_162); +return x_164; } else { -lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; -x_159 = lean_ctor_get(x_154, 0); -lean_inc(x_159); -x_160 = lean_ctor_get(x_154, 1); -lean_inc(x_160); -if (lean_is_exclusive(x_154)) { - lean_ctor_release(x_154, 0); - lean_ctor_release(x_154, 1); - x_161 = x_154; +lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; +x_165 = lean_ctor_get(x_160, 0); +lean_inc(x_165); +x_166 = lean_ctor_get(x_160, 1); +lean_inc(x_166); +if (lean_is_exclusive(x_160)) { + lean_ctor_release(x_160, 0); + lean_ctor_release(x_160, 1); + x_167 = x_160; } else { - lean_dec_ref(x_154); - x_161 = lean_box(0); + lean_dec_ref(x_160); + x_167 = lean_box(0); } -if (lean_is_scalar(x_161)) { - x_162 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_167)) { + x_168 = lean_alloc_ctor(1, 2, 0); } else { - x_162 = x_161; + x_168 = x_167; } -lean_ctor_set(x_162, 0, x_159); -lean_ctor_set(x_162, 1, x_160); -return x_162; +lean_ctor_set(x_168, 0, x_165); +lean_ctor_set(x_168, 1, x_166); +return x_168; } } else { -lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; -if (lean_is_exclusive(x_146)) { - lean_ctor_release(x_146, 0); - lean_ctor_release(x_146, 1); - x_163 = x_146; +lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; +if (lean_is_exclusive(x_151)) { + lean_ctor_release(x_151, 0); + lean_ctor_release(x_151, 1); + x_169 = x_151; } else { - lean_dec_ref(x_146); - x_163 = lean_box(0); + lean_dec_ref(x_151); + x_169 = lean_box(0); } -x_164 = lean_ctor_get(x_149, 0); -lean_inc(x_164); -if (lean_is_exclusive(x_149)) { - lean_ctor_release(x_149, 0); - x_165 = x_149; +x_170 = lean_ctor_get(x_155, 0); +lean_inc(x_170); +if (lean_is_exclusive(x_155)) { + lean_ctor_release(x_155, 0); + x_171 = x_155; } else { - lean_dec_ref(x_149); - x_165 = lean_box(0); + lean_dec_ref(x_155); + x_171 = lean_box(0); } -x_166 = lean_io_promise_new(x_8); -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; uint8_t x_172; lean_object* x_173; -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); -lean_inc(x_167); -x_169 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_parseCmd___lambda__6), 6, 4); -lean_closure_set(x_169, 0, x_144); -lean_closure_set(x_169, 1, x_167); -lean_closure_set(x_169, 2, x_3); -lean_closure_set(x_169, 3, x_164); -x_170 = lean_ctor_get(x_148, 4); -lean_inc(x_170); -x_171 = lean_ctor_get(x_170, 0); -lean_inc(x_171); -x_172 = 0; -x_173 = l_Lean_Language_SnapshotTask_bindIO___rarg(x_170, x_169, x_171, x_172, x_168); -if (lean_obj_tag(x_173) == 0) +x_172 = lean_io_promise_new(x_9); +if (lean_obj_tag(x_172) == 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; -x_174 = lean_ctor_get(x_173, 1); +lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; uint8_t x_179; lean_object* x_180; +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_173); -x_175 = lean_box(0); -x_176 = lean_io_promise_result(x_167); -x_177 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_177, 0, x_175); -lean_ctor_set(x_177, 1, x_176); -if (lean_is_scalar(x_165)) { - x_178 = lean_alloc_ctor(1, 1, 0); -} else { - x_178 = x_165; -} -lean_ctor_set(x_178, 0, x_177); -if (lean_is_scalar(x_163)) { - x_179 = lean_alloc_ctor(0, 2, 0); -} else { - x_179 = x_163; -} -lean_ctor_set(x_179, 0, x_148); -lean_ctor_set(x_179, 1, x_178); -x_180 = lean_io_promise_resolve(x_179, x_4, x_174); -lean_dec(x_4); +lean_dec(x_172); +x_175 = lean_box(x_4); +lean_inc(x_173); +x_176 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_parseCmd___lambda__8___boxed), 7, 5); +lean_closure_set(x_176, 0, x_149); +lean_closure_set(x_176, 1, x_173); +lean_closure_set(x_176, 2, x_175); +lean_closure_set(x_176, 3, x_3); +lean_closure_set(x_176, 4, x_170); +x_177 = lean_ctor_get(x_154, 4); +lean_inc(x_177); +x_178 = lean_ctor_get(x_177, 0); +lean_inc(x_178); +x_179 = 1; +x_180 = l_Lean_Language_SnapshotTask_bindIO___rarg(x_177, x_176, x_178, x_179, x_174); if (lean_obj_tag(x_180) == 0) { -lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; -x_181 = lean_ctor_get(x_180, 0); +lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; +x_181 = lean_ctor_get(x_180, 1); lean_inc(x_181); -x_182 = lean_ctor_get(x_180, 1); -lean_inc(x_182); -if (lean_is_exclusive(x_180)) { - lean_ctor_release(x_180, 0); - lean_ctor_release(x_180, 1); - x_183 = x_180; +lean_dec(x_180); +x_182 = lean_box(0); +x_183 = lean_io_promise_result(x_173); +x_184 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_184, 0, x_182); +lean_ctor_set(x_184, 1, x_183); +if (lean_is_scalar(x_171)) { + x_185 = lean_alloc_ctor(1, 1, 0); +} else { + x_185 = x_171; +} +lean_ctor_set(x_185, 0, x_184); +if (lean_is_scalar(x_169)) { + x_186 = lean_alloc_ctor(0, 2, 0); +} else { + x_186 = x_169; +} +lean_ctor_set(x_186, 0, x_154); +lean_ctor_set(x_186, 1, x_185); +x_187 = lean_io_promise_resolve(x_186, x_5, x_181); +lean_dec(x_5); +if (lean_obj_tag(x_187) == 0) +{ +lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; +x_188 = lean_ctor_get(x_187, 0); +lean_inc(x_188); +x_189 = lean_ctor_get(x_187, 1); +lean_inc(x_189); +if (lean_is_exclusive(x_187)) { + lean_ctor_release(x_187, 0); + lean_ctor_release(x_187, 1); + x_190 = x_187; } else { - lean_dec_ref(x_180); - x_183 = lean_box(0); + lean_dec_ref(x_187); + x_190 = lean_box(0); } -if (lean_is_scalar(x_183)) { - x_184 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_190)) { + x_191 = lean_alloc_ctor(0, 2, 0); } else { - x_184 = x_183; + x_191 = x_190; } -lean_ctor_set(x_184, 0, x_181); -lean_ctor_set(x_184, 1, x_182); -return x_184; +lean_ctor_set(x_191, 0, x_188); +lean_ctor_set(x_191, 1, x_189); +return x_191; } else { -lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; -x_185 = lean_ctor_get(x_180, 0); -lean_inc(x_185); -x_186 = lean_ctor_get(x_180, 1); -lean_inc(x_186); -if (lean_is_exclusive(x_180)) { - lean_ctor_release(x_180, 0); - lean_ctor_release(x_180, 1); - x_187 = x_180; +lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; +x_192 = lean_ctor_get(x_187, 0); +lean_inc(x_192); +x_193 = lean_ctor_get(x_187, 1); +lean_inc(x_193); +if (lean_is_exclusive(x_187)) { + lean_ctor_release(x_187, 0); + lean_ctor_release(x_187, 1); + x_194 = x_187; } else { - lean_dec_ref(x_180); - x_187 = lean_box(0); + lean_dec_ref(x_187); + x_194 = lean_box(0); } -if (lean_is_scalar(x_187)) { - x_188 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_194)) { + x_195 = lean_alloc_ctor(1, 2, 0); } else { - x_188 = x_187; + x_195 = x_194; } -lean_ctor_set(x_188, 0, x_185); -lean_ctor_set(x_188, 1, x_186); -return x_188; +lean_ctor_set(x_195, 0, x_192); +lean_ctor_set(x_195, 1, x_193); +return x_195; } } else { -lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; -lean_dec(x_167); -lean_dec(x_165); -lean_dec(x_163); -lean_dec(x_148); -lean_dec(x_4); -x_189 = lean_ctor_get(x_173, 0); -lean_inc(x_189); -x_190 = lean_ctor_get(x_173, 1); -lean_inc(x_190); -if (lean_is_exclusive(x_173)) { - lean_ctor_release(x_173, 0); - lean_ctor_release(x_173, 1); - x_191 = x_173; +lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; +lean_dec(x_173); +lean_dec(x_171); +lean_dec(x_169); +lean_dec(x_154); +lean_dec(x_5); +x_196 = lean_ctor_get(x_180, 0); +lean_inc(x_196); +x_197 = lean_ctor_get(x_180, 1); +lean_inc(x_197); +if (lean_is_exclusive(x_180)) { + lean_ctor_release(x_180, 0); + lean_ctor_release(x_180, 1); + x_198 = x_180; } else { - lean_dec_ref(x_173); - x_191 = lean_box(0); + lean_dec_ref(x_180); + x_198 = lean_box(0); } -if (lean_is_scalar(x_191)) { - x_192 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_198)) { + x_199 = lean_alloc_ctor(1, 2, 0); } else { - x_192 = x_191; + x_199 = x_198; } -lean_ctor_set(x_192, 0, x_189); -lean_ctor_set(x_192, 1, x_190); -return x_192; +lean_ctor_set(x_199, 0, x_196); +lean_ctor_set(x_199, 1, x_197); +return x_199; } } else { -lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; -lean_dec(x_165); -lean_dec(x_164); -lean_dec(x_163); -lean_dec(x_148); -lean_dec(x_144); -lean_dec(x_4); +lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; +lean_dec(x_171); +lean_dec(x_170); +lean_dec(x_169); +lean_dec(x_154); +lean_dec(x_149); +lean_dec(x_5); lean_dec(x_3); -x_193 = lean_ctor_get(x_166, 0); -lean_inc(x_193); -x_194 = lean_ctor_get(x_166, 1); -lean_inc(x_194); -if (lean_is_exclusive(x_166)) { - lean_ctor_release(x_166, 0); - lean_ctor_release(x_166, 1); - x_195 = x_166; +x_200 = lean_ctor_get(x_172, 0); +lean_inc(x_200); +x_201 = lean_ctor_get(x_172, 1); +lean_inc(x_201); +if (lean_is_exclusive(x_172)) { + lean_ctor_release(x_172, 0); + lean_ctor_release(x_172, 1); + x_202 = x_172; } else { - lean_dec_ref(x_166); - x_195 = lean_box(0); + lean_dec_ref(x_172); + x_202 = lean_box(0); } -if (lean_is_scalar(x_195)) { - x_196 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_202)) { + x_203 = lean_alloc_ctor(1, 2, 0); } else { - x_196 = x_195; + x_203 = x_202; } -lean_ctor_set(x_196, 0, x_193); -lean_ctor_set(x_196, 1, x_194); -return x_196; +lean_ctor_set(x_203, 0, x_200); +lean_ctor_set(x_203, 1, x_201); +return x_203; } } } @@ -6545,140 +7191,145 @@ return x_196; } } } -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___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_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, lean_object* x_6, lean_object* x_7) { _start: { -if (lean_obj_tag(x_5) == 0) +if (lean_obj_tag(x_1) == 0) { -lean_object* x_9; lean_object* x_10; -x_9 = lean_box(0); -x_10 = l_Lean_Language_Lean_process_parseCmd___lambda__7(x_1, x_2, x_3, x_4, x_5, x_9, x_7, x_8); -return x_10; +lean_object* x_8; lean_object* x_9; +x_8 = lean_box(0); +lean_inc(x_6); +x_9 = l_Lean_Language_Lean_process_parseCmd___lambda__9(x_2, x_3, x_6, x_5, x_4, x_1, x_8, x_6, x_7); +return x_9; } else { -lean_object* x_11; lean_object* x_12; -x_11 = lean_ctor_get(x_5, 0); +lean_object* x_10; lean_object* x_11; +x_10 = lean_ctor_get(x_1, 0); +lean_inc(x_10); +x_11 = lean_ctor_get(x_10, 1); lean_inc(x_11); -x_12 = lean_ctor_get(x_11, 1); -lean_inc(x_12); -if (lean_obj_tag(x_12) == 0) +if (lean_obj_tag(x_11) == 0) { -lean_object* x_13; lean_object* x_14; -lean_dec(x_11); -x_13 = lean_box(0); -x_14 = l_Lean_Language_Lean_process_parseCmd___lambda__7(x_1, x_2, x_3, x_4, x_5, x_13, x_7, x_8); -return x_14; +lean_object* x_12; lean_object* x_13; +lean_dec(x_10); +x_12 = lean_box(0); +lean_inc(x_6); +x_13 = l_Lean_Language_Lean_process_parseCmd___lambda__9(x_2, x_3, x_6, x_5, x_4, x_1, x_12, x_6, x_7); +return x_13; } else { -lean_object* x_15; lean_object* x_16; lean_object* x_17; +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_ctor_get(x_11, 0); lean_inc(x_15); lean_dec(x_11); -x_16 = lean_ctor_get(x_12, 0); -lean_inc(x_16); -lean_dec(x_12); -lean_inc(x_16); -x_17 = l_Lean_Language_SnapshotTask_get_x3f___rarg(x_16, x_8); +lean_inc(x_15); +x_16 = l_Lean_Language_SnapshotTask_get_x3f___rarg(x_15, x_7); +if (lean_obj_tag(x_16) == 0) +{ +lean_object* x_17; +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); if (lean_obj_tag(x_17) == 0) { -lean_object* x_18; -x_18 = lean_ctor_get(x_17, 0); +lean_object* x_18; lean_object* x_19; lean_object* x_20; +lean_dec(x_15); +lean_dec(x_14); +x_18 = lean_ctor_get(x_16, 1); lean_inc(x_18); -if (lean_obj_tag(x_18) == 0) -{ -lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_dec(x_16); -lean_dec(x_15); -x_19 = lean_ctor_get(x_17, 1); -lean_inc(x_19); -lean_dec(x_17); -x_20 = lean_box(0); -x_21 = l_Lean_Language_Lean_process_parseCmd___lambda__7(x_1, x_2, x_3, x_4, x_5, x_20, x_7, x_19); -return x_21; +x_19 = lean_box(0); +lean_inc(x_6); +x_20 = l_Lean_Language_Lean_process_parseCmd___lambda__9(x_2, x_3, x_6, x_5, x_4, x_1, x_19, x_6, x_18); +return x_20; } else { -uint8_t x_22; -x_22 = !lean_is_exclusive(x_18); -if (x_22 == 0) +uint8_t x_21; +x_21 = !lean_is_exclusive(x_17); +if (x_21 == 0) { -lean_object* x_23; lean_object* x_24; uint8_t x_25; -x_23 = lean_ctor_get(x_18, 0); -x_24 = lean_ctor_get(x_17, 1); -lean_inc(x_24); -lean_dec(x_17); -x_25 = !lean_is_exclusive(x_23); -if (x_25 == 0) +lean_object* x_22; lean_object* x_23; uint8_t x_24; +x_22 = lean_ctor_get(x_17, 0); +x_23 = lean_ctor_get(x_16, 1); +lean_inc(x_23); +lean_dec(x_16); +x_24 = !lean_is_exclusive(x_22); +if (x_24 == 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; uint8_t x_32; -x_26 = lean_ctor_get(x_23, 0); -x_27 = lean_ctor_get(x_23, 1); -lean_dec(x_27); -x_28 = lean_ctor_get(x_26, 2); -lean_inc(x_28); +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_22, 0); +x_26 = lean_ctor_get(x_22, 1); lean_dec(x_26); -x_29 = lean_ctor_get(x_28, 0); -lean_inc(x_29); +x_27 = lean_ctor_get(x_25, 2); +lean_inc(x_27); +lean_dec(x_25); +x_28 = lean_ctor_get(x_27, 0); +lean_inc(x_28); +lean_dec(x_27); +x_29 = l_Lean_Language_Lean_isBeforeEditPos(x_28, x_6, x_23); lean_dec(x_28); -x_30 = l_Lean_Language_Lean_isBeforeEditPos(x_29, x_7, x_24); -lean_dec(x_29); -x_31 = lean_ctor_get(x_30, 0); -lean_inc(x_31); -x_32 = lean_unbox(x_31); -lean_dec(x_31); -if (x_32 == 0) +x_30 = lean_ctor_get(x_29, 0); +lean_inc(x_30); +x_31 = lean_unbox(x_30); +lean_dec(x_30); +if (x_31 == 0) { -lean_object* x_33; lean_object* x_34; lean_object* x_35; -lean_free_object(x_23); -lean_free_object(x_18); -lean_dec(x_16); +lean_object* x_32; lean_object* x_33; lean_object* x_34; +lean_free_object(x_22); +lean_free_object(x_17); lean_dec(x_15); -x_33 = lean_ctor_get(x_30, 1); -lean_inc(x_33); -lean_dec(x_30); -x_34 = lean_box(0); -x_35 = l_Lean_Language_Lean_process_parseCmd___lambda__7(x_1, x_2, x_3, x_4, x_5, x_34, x_7, x_33); -return x_35; +lean_dec(x_14); +x_32 = lean_ctor_get(x_29, 1); +lean_inc(x_32); +lean_dec(x_29); +x_33 = lean_box(0); +lean_inc(x_6); +x_34 = l_Lean_Language_Lean_process_parseCmd___lambda__9(x_2, x_3, x_6, x_5, x_4, x_1, x_33, x_6, x_32); +return x_34; } else { -uint8_t x_36; -lean_dec(x_7); -lean_dec(x_5); +uint8_t x_35; +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_36 = !lean_is_exclusive(x_30); -if (x_36 == 0) +x_35 = !lean_is_exclusive(x_29); +if (x_35 == 0) { -lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_37 = lean_ctor_get(x_30, 1); -x_38 = lean_ctor_get(x_30, 0); -lean_dec(x_38); -x_39 = lean_ctor_get(x_15, 2); -lean_inc(x_39); -x_40 = lean_io_promise_new(x_37); -if (lean_obj_tag(x_40) == 0) +lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_36 = lean_ctor_get(x_29, 1); +x_37 = lean_ctor_get(x_29, 0); +lean_dec(x_37); +x_38 = lean_ctor_get(x_14, 2); +lean_inc(x_38); +x_39 = lean_io_promise_new(x_36); +if (lean_obj_tag(x_39) == 0) { -lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; uint8_t x_46; lean_object* x_47; -x_41 = lean_ctor_get(x_40, 0); -lean_inc(x_41); -x_42 = lean_ctor_get(x_40, 1); -lean_inc(x_42); -lean_dec(x_40); +lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; uint8_t x_46; lean_object* x_47; +x_40 = lean_ctor_get(x_39, 0); +lean_inc(x_40); +x_41 = lean_ctor_get(x_39, 1); lean_inc(x_41); -x_43 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_parseCmd___lambda__6), 6, 4); -lean_closure_set(x_43, 0, x_39); -lean_closure_set(x_43, 1, x_41); -lean_closure_set(x_43, 2, x_3); -lean_closure_set(x_43, 3, x_16); -x_44 = lean_ctor_get(x_15, 4); +lean_dec(x_39); +x_42 = lean_box(x_5); +lean_inc(x_40); +x_43 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_parseCmd___lambda__8___boxed), 7, 5); +lean_closure_set(x_43, 0, x_38); +lean_closure_set(x_43, 1, x_40); +lean_closure_set(x_43, 2, x_42); +lean_closure_set(x_43, 3, x_6); +lean_closure_set(x_43, 4, x_15); +x_44 = lean_ctor_get(x_14, 4); lean_inc(x_44); x_45 = lean_ctor_get(x_44, 0); lean_inc(x_45); -x_46 = 0; -x_47 = l_Lean_Language_SnapshotTask_bindIO___rarg(x_44, x_43, x_45, x_46, x_42); +x_46 = 1; +x_47 = l_Lean_Language_SnapshotTask_bindIO___rarg(x_44, x_43, x_45, x_46, x_41); if (lean_obj_tag(x_47) == 0) { lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; @@ -6686,13 +7337,13 @@ x_48 = lean_ctor_get(x_47, 1); lean_inc(x_48); lean_dec(x_47); x_49 = lean_box(0); -x_50 = lean_io_promise_result(x_41); -lean_ctor_set(x_30, 1, x_50); -lean_ctor_set(x_30, 0, x_49); -lean_ctor_set(x_18, 0, x_30); -lean_ctor_set(x_23, 1, x_18); -lean_ctor_set(x_23, 0, x_15); -x_51 = lean_io_promise_resolve(x_23, x_4, x_48); +x_50 = lean_io_promise_result(x_40); +lean_ctor_set(x_29, 1, x_50); +lean_ctor_set(x_29, 0, x_49); +lean_ctor_set(x_17, 0, x_29); +lean_ctor_set(x_22, 1, x_17); +lean_ctor_set(x_22, 0, x_14); +x_51 = lean_io_promise_resolve(x_22, x_4, x_48); lean_dec(x_4); if (lean_obj_tag(x_51) == 0) { @@ -6742,11 +7393,11 @@ return x_59; else { uint8_t x_60; -lean_dec(x_41); -lean_free_object(x_30); -lean_free_object(x_23); -lean_free_object(x_18); -lean_dec(x_15); +lean_dec(x_40); +lean_free_object(x_29); +lean_free_object(x_22); +lean_free_object(x_17); +lean_dec(x_14); lean_dec(x_4); x_60 = !lean_is_exclusive(x_47); if (x_60 == 0) @@ -6771,27 +7422,27 @@ return x_63; else { uint8_t x_64; -lean_dec(x_39); -lean_free_object(x_30); -lean_free_object(x_23); -lean_free_object(x_18); -lean_dec(x_16); +lean_dec(x_38); +lean_free_object(x_29); +lean_free_object(x_22); +lean_free_object(x_17); lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_6); lean_dec(x_4); -lean_dec(x_3); -x_64 = !lean_is_exclusive(x_40); +x_64 = !lean_is_exclusive(x_39); if (x_64 == 0) { -return x_40; +return x_39; } else { lean_object* x_65; lean_object* x_66; lean_object* x_67; -x_65 = lean_ctor_get(x_40, 0); -x_66 = lean_ctor_get(x_40, 1); +x_65 = lean_ctor_get(x_39, 0); +x_66 = lean_ctor_get(x_39, 1); lean_inc(x_66); lean_inc(x_65); -lean_dec(x_40); +lean_dec(x_39); x_67 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_67, 0, x_65); lean_ctor_set(x_67, 1, x_66); @@ -6802,824 +7453,625 @@ return x_67; else { lean_object* x_68; lean_object* x_69; lean_object* x_70; -x_68 = lean_ctor_get(x_30, 1); +x_68 = lean_ctor_get(x_29, 1); lean_inc(x_68); -lean_dec(x_30); -x_69 = lean_ctor_get(x_15, 2); +lean_dec(x_29); +x_69 = lean_ctor_get(x_14, 2); lean_inc(x_69); x_70 = lean_io_promise_new(x_68); if (lean_obj_tag(x_70) == 0) { -lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; uint8_t x_76; lean_object* x_77; +lean_object* x_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; x_71 = lean_ctor_get(x_70, 0); lean_inc(x_71); x_72 = lean_ctor_get(x_70, 1); lean_inc(x_72); lean_dec(x_70); +x_73 = lean_box(x_5); lean_inc(x_71); -x_73 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_parseCmd___lambda__6), 6, 4); -lean_closure_set(x_73, 0, x_69); -lean_closure_set(x_73, 1, x_71); -lean_closure_set(x_73, 2, x_3); -lean_closure_set(x_73, 3, x_16); -x_74 = lean_ctor_get(x_15, 4); -lean_inc(x_74); -x_75 = lean_ctor_get(x_74, 0); +x_74 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_parseCmd___lambda__8___boxed), 7, 5); +lean_closure_set(x_74, 0, x_69); +lean_closure_set(x_74, 1, x_71); +lean_closure_set(x_74, 2, x_73); +lean_closure_set(x_74, 3, x_6); +lean_closure_set(x_74, 4, x_15); +x_75 = lean_ctor_get(x_14, 4); lean_inc(x_75); -x_76 = 0; -x_77 = l_Lean_Language_SnapshotTask_bindIO___rarg(x_74, x_73, x_75, x_76, x_72); -if (lean_obj_tag(x_77) == 0) +x_76 = lean_ctor_get(x_75, 0); +lean_inc(x_76); +x_77 = 1; +x_78 = l_Lean_Language_SnapshotTask_bindIO___rarg(x_75, x_74, x_76, x_77, x_72); +if (lean_obj_tag(x_78) == 0) { -lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; -x_78 = lean_ctor_get(x_77, 1); -lean_inc(x_78); -lean_dec(x_77); -x_79 = lean_box(0); -x_80 = lean_io_promise_result(x_71); -x_81 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_81, 0, x_79); -lean_ctor_set(x_81, 1, x_80); -lean_ctor_set(x_18, 0, x_81); -lean_ctor_set(x_23, 1, x_18); -lean_ctor_set(x_23, 0, x_15); -x_82 = lean_io_promise_resolve(x_23, x_4, x_78); +lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; +x_79 = lean_ctor_get(x_78, 1); +lean_inc(x_79); +lean_dec(x_78); +x_80 = lean_box(0); +x_81 = lean_io_promise_result(x_71); +x_82 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_82, 0, x_80); +lean_ctor_set(x_82, 1, x_81); +lean_ctor_set(x_17, 0, x_82); +lean_ctor_set(x_22, 1, x_17); +lean_ctor_set(x_22, 0, x_14); +x_83 = lean_io_promise_resolve(x_22, x_4, x_79); lean_dec(x_4); -if (lean_obj_tag(x_82) == 0) +if (lean_obj_tag(x_83) == 0) { -lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; -x_83 = lean_ctor_get(x_82, 0); -lean_inc(x_83); -x_84 = lean_ctor_get(x_82, 1); +lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; +x_84 = lean_ctor_get(x_83, 0); lean_inc(x_84); -if (lean_is_exclusive(x_82)) { - lean_ctor_release(x_82, 0); - lean_ctor_release(x_82, 1); - x_85 = x_82; +x_85 = lean_ctor_get(x_83, 1); +lean_inc(x_85); +if (lean_is_exclusive(x_83)) { + lean_ctor_release(x_83, 0); + lean_ctor_release(x_83, 1); + x_86 = x_83; } else { - lean_dec_ref(x_82); - x_85 = lean_box(0); + lean_dec_ref(x_83); + x_86 = lean_box(0); } -if (lean_is_scalar(x_85)) { - x_86 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_86)) { + x_87 = lean_alloc_ctor(0, 2, 0); } else { - x_86 = x_85; + x_87 = x_86; } -lean_ctor_set(x_86, 0, x_83); -lean_ctor_set(x_86, 1, x_84); -return x_86; +lean_ctor_set(x_87, 0, x_84); +lean_ctor_set(x_87, 1, x_85); +return x_87; } else { -lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; -x_87 = lean_ctor_get(x_82, 0); -lean_inc(x_87); -x_88 = lean_ctor_get(x_82, 1); +lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; +x_88 = lean_ctor_get(x_83, 0); lean_inc(x_88); -if (lean_is_exclusive(x_82)) { - lean_ctor_release(x_82, 0); - lean_ctor_release(x_82, 1); - x_89 = x_82; +x_89 = lean_ctor_get(x_83, 1); +lean_inc(x_89); +if (lean_is_exclusive(x_83)) { + lean_ctor_release(x_83, 0); + lean_ctor_release(x_83, 1); + x_90 = x_83; } else { - lean_dec_ref(x_82); - x_89 = lean_box(0); + lean_dec_ref(x_83); + x_90 = lean_box(0); } -if (lean_is_scalar(x_89)) { - x_90 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_90)) { + x_91 = lean_alloc_ctor(1, 2, 0); } else { - x_90 = x_89; + x_91 = x_90; } -lean_ctor_set(x_90, 0, x_87); -lean_ctor_set(x_90, 1, x_88); -return x_90; +lean_ctor_set(x_91, 0, x_88); +lean_ctor_set(x_91, 1, x_89); +return x_91; } } else { -lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; +lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_dec(x_71); -lean_free_object(x_23); -lean_free_object(x_18); -lean_dec(x_15); +lean_free_object(x_22); +lean_free_object(x_17); +lean_dec(x_14); lean_dec(x_4); -x_91 = lean_ctor_get(x_77, 0); -lean_inc(x_91); -x_92 = lean_ctor_get(x_77, 1); +x_92 = lean_ctor_get(x_78, 0); lean_inc(x_92); -if (lean_is_exclusive(x_77)) { - lean_ctor_release(x_77, 0); - lean_ctor_release(x_77, 1); - x_93 = x_77; +x_93 = lean_ctor_get(x_78, 1); +lean_inc(x_93); +if (lean_is_exclusive(x_78)) { + lean_ctor_release(x_78, 0); + lean_ctor_release(x_78, 1); + x_94 = x_78; } else { - lean_dec_ref(x_77); - x_93 = lean_box(0); + lean_dec_ref(x_78); + x_94 = lean_box(0); } -if (lean_is_scalar(x_93)) { - x_94 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_94)) { + x_95 = lean_alloc_ctor(1, 2, 0); } else { - x_94 = x_93; + x_95 = x_94; } -lean_ctor_set(x_94, 0, x_91); -lean_ctor_set(x_94, 1, x_92); -return x_94; +lean_ctor_set(x_95, 0, x_92); +lean_ctor_set(x_95, 1, x_93); +return x_95; } } else { -lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; +lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_dec(x_69); -lean_free_object(x_23); -lean_free_object(x_18); -lean_dec(x_16); +lean_free_object(x_22); +lean_free_object(x_17); lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_6); lean_dec(x_4); -lean_dec(x_3); -x_95 = lean_ctor_get(x_70, 0); -lean_inc(x_95); -x_96 = lean_ctor_get(x_70, 1); +x_96 = lean_ctor_get(x_70, 0); lean_inc(x_96); +x_97 = lean_ctor_get(x_70, 1); +lean_inc(x_97); if (lean_is_exclusive(x_70)) { lean_ctor_release(x_70, 0); lean_ctor_release(x_70, 1); - x_97 = x_70; + x_98 = x_70; } else { lean_dec_ref(x_70); - x_97 = lean_box(0); + x_98 = lean_box(0); } -if (lean_is_scalar(x_97)) { - x_98 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_98)) { + x_99 = lean_alloc_ctor(1, 2, 0); } else { - x_98 = x_97; + x_99 = x_98; } -lean_ctor_set(x_98, 0, x_95); -lean_ctor_set(x_98, 1, x_96); -return x_98; +lean_ctor_set(x_99, 0, x_96); +lean_ctor_set(x_99, 1, x_97); +return x_99; } } } } else { -lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; uint8_t x_104; -x_99 = lean_ctor_get(x_23, 0); -lean_inc(x_99); -lean_dec(x_23); -x_100 = lean_ctor_get(x_99, 2); +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_22, 0); lean_inc(x_100); -lean_dec(x_99); -x_101 = lean_ctor_get(x_100, 0); +lean_dec(x_22); +x_101 = lean_ctor_get(x_100, 2); lean_inc(x_101); lean_dec(x_100); -x_102 = l_Lean_Language_Lean_isBeforeEditPos(x_101, x_7, x_24); +x_102 = lean_ctor_get(x_101, 0); +lean_inc(x_102); lean_dec(x_101); -x_103 = lean_ctor_get(x_102, 0); -lean_inc(x_103); -x_104 = lean_unbox(x_103); -lean_dec(x_103); -if (x_104 == 0) -{ -lean_object* x_105; lean_object* x_106; lean_object* x_107; -lean_free_object(x_18); -lean_dec(x_16); -lean_dec(x_15); -x_105 = lean_ctor_get(x_102, 1); -lean_inc(x_105); +x_103 = l_Lean_Language_Lean_isBeforeEditPos(x_102, x_6, x_23); lean_dec(x_102); -x_106 = lean_box(0); -x_107 = l_Lean_Language_Lean_process_parseCmd___lambda__7(x_1, x_2, x_3, x_4, x_5, x_106, x_7, x_105); -return x_107; -} -else -{ -lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; -lean_dec(x_7); -lean_dec(x_5); -lean_dec(x_2); -lean_dec(x_1); -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; -} else { - lean_dec_ref(x_102); - x_109 = lean_box(0); -} -x_110 = lean_ctor_get(x_15, 2); -lean_inc(x_110); -x_111 = lean_io_promise_new(x_108); -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; uint8_t x_117; lean_object* x_118; -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_112); -x_114 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_parseCmd___lambda__6), 6, 4); -lean_closure_set(x_114, 0, x_110); -lean_closure_set(x_114, 1, x_112); -lean_closure_set(x_114, 2, x_3); -lean_closure_set(x_114, 3, x_16); -x_115 = lean_ctor_get(x_15, 4); -lean_inc(x_115); -x_116 = lean_ctor_get(x_115, 0); -lean_inc(x_116); -x_117 = 0; -x_118 = l_Lean_Language_SnapshotTask_bindIO___rarg(x_115, x_114, x_116, x_117, x_113); -if (lean_obj_tag(x_118) == 0) -{ -lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; -x_119 = lean_ctor_get(x_118, 1); -lean_inc(x_119); -lean_dec(x_118); -x_120 = lean_box(0); -x_121 = lean_io_promise_result(x_112); -if (lean_is_scalar(x_109)) { - x_122 = lean_alloc_ctor(0, 2, 0); -} else { - x_122 = x_109; -} -lean_ctor_set(x_122, 0, x_120); -lean_ctor_set(x_122, 1, x_121); -lean_ctor_set(x_18, 0, x_122); -x_123 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_123, 0, x_15); -lean_ctor_set(x_123, 1, x_18); -x_124 = lean_io_promise_resolve(x_123, x_4, x_119); -lean_dec(x_4); -if (lean_obj_tag(x_124) == 0) -{ -lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; -x_125 = lean_ctor_get(x_124, 0); -lean_inc(x_125); -x_126 = lean_ctor_get(x_124, 1); -lean_inc(x_126); -if (lean_is_exclusive(x_124)) { - lean_ctor_release(x_124, 0); - lean_ctor_release(x_124, 1); - x_127 = x_124; -} else { - lean_dec_ref(x_124); - x_127 = lean_box(0); -} -if (lean_is_scalar(x_127)) { - x_128 = lean_alloc_ctor(0, 2, 0); -} else { - x_128 = x_127; -} -lean_ctor_set(x_128, 0, x_125); -lean_ctor_set(x_128, 1, x_126); -return x_128; -} -else -{ -lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; -x_129 = lean_ctor_get(x_124, 0); -lean_inc(x_129); -x_130 = lean_ctor_get(x_124, 1); -lean_inc(x_130); -if (lean_is_exclusive(x_124)) { - lean_ctor_release(x_124, 0); - lean_ctor_release(x_124, 1); - x_131 = x_124; -} else { - lean_dec_ref(x_124); - x_131 = lean_box(0); -} -if (lean_is_scalar(x_131)) { - x_132 = lean_alloc_ctor(1, 2, 0); -} else { - x_132 = x_131; -} -lean_ctor_set(x_132, 0, x_129); -lean_ctor_set(x_132, 1, x_130); -return x_132; -} -} -else +x_104 = lean_ctor_get(x_103, 0); +lean_inc(x_104); +x_105 = lean_unbox(x_104); +lean_dec(x_104); +if (x_105 == 0) { -lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; -lean_dec(x_112); -lean_dec(x_109); -lean_free_object(x_18); +lean_object* x_106; lean_object* x_107; lean_object* x_108; +lean_free_object(x_17); lean_dec(x_15); -lean_dec(x_4); -x_133 = lean_ctor_get(x_118, 0); -lean_inc(x_133); -x_134 = lean_ctor_get(x_118, 1); -lean_inc(x_134); -if (lean_is_exclusive(x_118)) { - lean_ctor_release(x_118, 0); - lean_ctor_release(x_118, 1); - x_135 = x_118; -} else { - lean_dec_ref(x_118); - x_135 = lean_box(0); -} -if (lean_is_scalar(x_135)) { - x_136 = lean_alloc_ctor(1, 2, 0); -} else { - x_136 = x_135; -} -lean_ctor_set(x_136, 0, x_133); -lean_ctor_set(x_136, 1, x_134); -return x_136; -} +lean_dec(x_14); +x_106 = lean_ctor_get(x_103, 1); +lean_inc(x_106); +lean_dec(x_103); +x_107 = lean_box(0); +lean_inc(x_6); +x_108 = l_Lean_Language_Lean_process_parseCmd___lambda__9(x_2, x_3, x_6, x_5, x_4, x_1, x_107, x_6, x_106); +return x_108; } else { -lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; -lean_dec(x_110); -lean_dec(x_109); -lean_free_object(x_18); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_4); +lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_dec(x_3); -x_137 = lean_ctor_get(x_111, 0); -lean_inc(x_137); -x_138 = lean_ctor_get(x_111, 1); -lean_inc(x_138); -if (lean_is_exclusive(x_111)) { - lean_ctor_release(x_111, 0); - lean_ctor_release(x_111, 1); - x_139 = x_111; -} else { - lean_dec_ref(x_111); - x_139 = lean_box(0); -} -if (lean_is_scalar(x_139)) { - x_140 = lean_alloc_ctor(1, 2, 0); -} else { - x_140 = x_139; -} -lean_ctor_set(x_140, 0, x_137); -lean_ctor_set(x_140, 1, x_138); -return x_140; -} -} -} -} -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; uint8_t x_149; -x_141 = lean_ctor_get(x_18, 0); -lean_inc(x_141); -lean_dec(x_18); -x_142 = lean_ctor_get(x_17, 1); -lean_inc(x_142); -lean_dec(x_17); -x_143 = lean_ctor_get(x_141, 0); -lean_inc(x_143); -if (lean_is_exclusive(x_141)) { - lean_ctor_release(x_141, 0); - lean_ctor_release(x_141, 1); - x_144 = x_141; -} else { - lean_dec_ref(x_141); - x_144 = lean_box(0); -} -x_145 = lean_ctor_get(x_143, 2); -lean_inc(x_145); -lean_dec(x_143); -x_146 = lean_ctor_get(x_145, 0); -lean_inc(x_146); -lean_dec(x_145); -x_147 = l_Lean_Language_Lean_isBeforeEditPos(x_146, x_7, x_142); -lean_dec(x_146); -x_148 = lean_ctor_get(x_147, 0); -lean_inc(x_148); -x_149 = lean_unbox(x_148); -lean_dec(x_148); -if (x_149 == 0) -{ -lean_object* x_150; lean_object* x_151; lean_object* x_152; -lean_dec(x_144); -lean_dec(x_16); -lean_dec(x_15); -x_150 = lean_ctor_get(x_147, 1); -lean_inc(x_150); -lean_dec(x_147); -x_151 = lean_box(0); -x_152 = l_Lean_Language_Lean_process_parseCmd___lambda__7(x_1, x_2, x_3, x_4, x_5, x_151, x_7, x_150); -return x_152; -} -else -{ -lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; -lean_dec(x_7); -lean_dec(x_5); lean_dec(x_2); lean_dec(x_1); -x_153 = lean_ctor_get(x_147, 1); -lean_inc(x_153); -if (lean_is_exclusive(x_147)) { - lean_ctor_release(x_147, 0); - lean_ctor_release(x_147, 1); - x_154 = x_147; +x_109 = lean_ctor_get(x_103, 1); +lean_inc(x_109); +if (lean_is_exclusive(x_103)) { + lean_ctor_release(x_103, 0); + lean_ctor_release(x_103, 1); + x_110 = x_103; } else { - lean_dec_ref(x_147); - x_154 = lean_box(0); + lean_dec_ref(x_103); + x_110 = lean_box(0); } -x_155 = lean_ctor_get(x_15, 2); -lean_inc(x_155); -x_156 = lean_io_promise_new(x_153); -if (lean_obj_tag(x_156) == 0) +x_111 = lean_ctor_get(x_14, 2); +lean_inc(x_111); +x_112 = lean_io_promise_new(x_109); +if (lean_obj_tag(x_112) == 0) { -lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; uint8_t x_162; lean_object* x_163; -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); -lean_inc(x_157); -x_159 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_parseCmd___lambda__6), 6, 4); -lean_closure_set(x_159, 0, x_155); -lean_closure_set(x_159, 1, x_157); -lean_closure_set(x_159, 2, x_3); -lean_closure_set(x_159, 3, x_16); -x_160 = lean_ctor_get(x_15, 4); -lean_inc(x_160); -x_161 = lean_ctor_get(x_160, 0); -lean_inc(x_161); -x_162 = 0; -x_163 = l_Lean_Language_SnapshotTask_bindIO___rarg(x_160, x_159, x_161, x_162, x_158); -if (lean_obj_tag(x_163) == 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; uint8_t x_119; lean_object* x_120; +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_box(x_5); +lean_inc(x_113); +x_116 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_parseCmd___lambda__8___boxed), 7, 5); +lean_closure_set(x_116, 0, x_111); +lean_closure_set(x_116, 1, x_113); +lean_closure_set(x_116, 2, x_115); +lean_closure_set(x_116, 3, x_6); +lean_closure_set(x_116, 4, x_15); +x_117 = lean_ctor_get(x_14, 4); +lean_inc(x_117); +x_118 = lean_ctor_get(x_117, 0); +lean_inc(x_118); +x_119 = 1; +x_120 = l_Lean_Language_SnapshotTask_bindIO___rarg(x_117, x_116, x_118, x_119, x_114); +if (lean_obj_tag(x_120) == 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; lean_object* x_170; -x_164 = lean_ctor_get(x_163, 1); -lean_inc(x_164); -lean_dec(x_163); -x_165 = lean_box(0); -x_166 = lean_io_promise_result(x_157); -if (lean_is_scalar(x_154)) { - x_167 = lean_alloc_ctor(0, 2, 0); -} else { - x_167 = x_154; -} -lean_ctor_set(x_167, 0, x_165); -lean_ctor_set(x_167, 1, x_166); -x_168 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_168, 0, x_167); -if (lean_is_scalar(x_144)) { - x_169 = lean_alloc_ctor(0, 2, 0); +lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; +x_121 = lean_ctor_get(x_120, 1); +lean_inc(x_121); +lean_dec(x_120); +x_122 = lean_box(0); +x_123 = lean_io_promise_result(x_113); +if (lean_is_scalar(x_110)) { + x_124 = lean_alloc_ctor(0, 2, 0); } else { - x_169 = x_144; + x_124 = x_110; } -lean_ctor_set(x_169, 0, x_15); -lean_ctor_set(x_169, 1, x_168); -x_170 = lean_io_promise_resolve(x_169, x_4, x_164); +lean_ctor_set(x_124, 0, x_122); +lean_ctor_set(x_124, 1, x_123); +lean_ctor_set(x_17, 0, x_124); +x_125 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_125, 0, x_14); +lean_ctor_set(x_125, 1, x_17); +x_126 = lean_io_promise_resolve(x_125, x_4, x_121); lean_dec(x_4); -if (lean_obj_tag(x_170) == 0) +if (lean_obj_tag(x_126) == 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_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_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; +x_127 = lean_ctor_get(x_126, 0); +lean_inc(x_127); +x_128 = lean_ctor_get(x_126, 1); +lean_inc(x_128); +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_170); - x_173 = lean_box(0); + lean_dec_ref(x_126); + x_129 = lean_box(0); } -if (lean_is_scalar(x_173)) { - x_174 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_129)) { + x_130 = lean_alloc_ctor(0, 2, 0); } else { - x_174 = x_173; + x_130 = x_129; } -lean_ctor_set(x_174, 0, x_171); -lean_ctor_set(x_174, 1, x_172); -return x_174; +lean_ctor_set(x_130, 0, x_127); +lean_ctor_set(x_130, 1, x_128); +return x_130; } else { -lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; -x_175 = lean_ctor_get(x_170, 0); -lean_inc(x_175); -x_176 = lean_ctor_get(x_170, 1); -lean_inc(x_176); -if (lean_is_exclusive(x_170)) { - lean_ctor_release(x_170, 0); - lean_ctor_release(x_170, 1); - x_177 = x_170; +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_170); - x_177 = lean_box(0); + lean_dec_ref(x_126); + x_133 = lean_box(0); } -if (lean_is_scalar(x_177)) { - x_178 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_133)) { + x_134 = lean_alloc_ctor(1, 2, 0); } else { - x_178 = x_177; + x_134 = x_133; } -lean_ctor_set(x_178, 0, x_175); -lean_ctor_set(x_178, 1, x_176); -return x_178; +lean_ctor_set(x_134, 0, x_131); +lean_ctor_set(x_134, 1, x_132); +return x_134; } } else { -lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; -lean_dec(x_157); -lean_dec(x_154); -lean_dec(x_144); -lean_dec(x_15); +lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; +lean_dec(x_113); +lean_dec(x_110); +lean_free_object(x_17); +lean_dec(x_14); lean_dec(x_4); -x_179 = lean_ctor_get(x_163, 0); -lean_inc(x_179); -x_180 = lean_ctor_get(x_163, 1); -lean_inc(x_180); -if (lean_is_exclusive(x_163)) { - lean_ctor_release(x_163, 0); - lean_ctor_release(x_163, 1); - x_181 = x_163; +x_135 = lean_ctor_get(x_120, 0); +lean_inc(x_135); +x_136 = lean_ctor_get(x_120, 1); +lean_inc(x_136); +if (lean_is_exclusive(x_120)) { + lean_ctor_release(x_120, 0); + lean_ctor_release(x_120, 1); + x_137 = x_120; } else { - lean_dec_ref(x_163); - x_181 = lean_box(0); + lean_dec_ref(x_120); + x_137 = lean_box(0); } -if (lean_is_scalar(x_181)) { - x_182 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_137)) { + x_138 = lean_alloc_ctor(1, 2, 0); } else { - x_182 = x_181; + x_138 = x_137; } -lean_ctor_set(x_182, 0, x_179); -lean_ctor_set(x_182, 1, x_180); -return x_182; +lean_ctor_set(x_138, 0, x_135); +lean_ctor_set(x_138, 1, x_136); +return x_138; } } else { -lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; -lean_dec(x_155); -lean_dec(x_154); -lean_dec(x_144); -lean_dec(x_16); +lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; +lean_dec(x_111); +lean_dec(x_110); +lean_free_object(x_17); lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_6); lean_dec(x_4); -lean_dec(x_3); -x_183 = lean_ctor_get(x_156, 0); -lean_inc(x_183); -x_184 = lean_ctor_get(x_156, 1); -lean_inc(x_184); -if (lean_is_exclusive(x_156)) { - lean_ctor_release(x_156, 0); - lean_ctor_release(x_156, 1); - x_185 = x_156; +x_139 = lean_ctor_get(x_112, 0); +lean_inc(x_139); +x_140 = lean_ctor_get(x_112, 1); +lean_inc(x_140); +if (lean_is_exclusive(x_112)) { + lean_ctor_release(x_112, 0); + lean_ctor_release(x_112, 1); + x_141 = x_112; } else { - lean_dec_ref(x_156); - x_185 = lean_box(0); + lean_dec_ref(x_112); + x_141 = lean_box(0); } -if (lean_is_scalar(x_185)) { - x_186 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_141)) { + x_142 = lean_alloc_ctor(1, 2, 0); } else { - x_186 = x_185; -} -lean_ctor_set(x_186, 0, x_183); -lean_ctor_set(x_186, 1, x_184); -return x_186; + x_142 = x_141; } +lean_ctor_set(x_142, 0, x_139); +lean_ctor_set(x_142, 1, x_140); +return x_142; } } } } else { -uint8_t x_187; +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; uint8_t x_151; +x_143 = lean_ctor_get(x_17, 0); +lean_inc(x_143); +lean_dec(x_17); +x_144 = lean_ctor_get(x_16, 1); +lean_inc(x_144); lean_dec(x_16); -lean_dec(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); -x_187 = !lean_is_exclusive(x_17); -if (x_187 == 0) +x_145 = lean_ctor_get(x_143, 0); +lean_inc(x_145); +if (lean_is_exclusive(x_143)) { + lean_ctor_release(x_143, 0); + lean_ctor_release(x_143, 1); + x_146 = x_143; +} else { + lean_dec_ref(x_143); + x_146 = lean_box(0); +} +x_147 = lean_ctor_get(x_145, 2); +lean_inc(x_147); +lean_dec(x_145); +x_148 = lean_ctor_get(x_147, 0); +lean_inc(x_148); +lean_dec(x_147); +x_149 = l_Lean_Language_Lean_isBeforeEditPos(x_148, x_6, x_144); +lean_dec(x_148); +x_150 = lean_ctor_get(x_149, 0); +lean_inc(x_150); +x_151 = lean_unbox(x_150); +lean_dec(x_150); +if (x_151 == 0) { -return x_17; +lean_object* x_152; lean_object* x_153; lean_object* x_154; +lean_dec(x_146); +lean_dec(x_15); +lean_dec(x_14); +x_152 = lean_ctor_get(x_149, 1); +lean_inc(x_152); +lean_dec(x_149); +x_153 = lean_box(0); +lean_inc(x_6); +x_154 = l_Lean_Language_Lean_process_parseCmd___lambda__9(x_2, x_3, x_6, x_5, x_4, x_1, x_153, x_6, x_152); +return x_154; } 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_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; -} -} -} -} -} +lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_155 = lean_ctor_get(x_149, 1); +lean_inc(x_155); +if (lean_is_exclusive(x_149)) { + lean_ctor_release(x_149, 0); + lean_ctor_release(x_149, 1); + x_156 = x_149; +} else { + lean_dec_ref(x_149); + x_156 = lean_box(0); } -static lean_object* _init_l_Lean_Language_Lean_process_parseCmd___closed__1() { -_start: +x_157 = lean_ctor_get(x_14, 2); +lean_inc(x_157); +x_158 = lean_io_promise_new(x_155); +if (lean_obj_tag(x_158) == 0) { -lean_object* x_1; lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; -x_1 = lean_box(0); -x_2 = l_Lean_Language_Lean_process_parseCmd___lambda__2___closed__3; -x_3 = l_Lean_Language_Snapshot_Diagnostics_empty; -x_4 = 0; -x_5 = lean_alloc_ctor(0, 3, 1); -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_uint8(x_5, sizeof(void*)*3, x_4); -return x_5; -} -} -static lean_object* _init_l_Lean_Language_Lean_process_parseCmd___closed__2() { -_start: +lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; uint8_t x_165; lean_object* x_166; +x_159 = lean_ctor_get(x_158, 0); +lean_inc(x_159); +x_160 = lean_ctor_get(x_158, 1); +lean_inc(x_160); +lean_dec(x_158); +x_161 = lean_box(x_5); +lean_inc(x_159); +x_162 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_parseCmd___lambda__8___boxed), 7, 5); +lean_closure_set(x_162, 0, x_157); +lean_closure_set(x_162, 1, x_159); +lean_closure_set(x_162, 2, x_161); +lean_closure_set(x_162, 3, x_6); +lean_closure_set(x_162, 4, x_15); +x_163 = lean_ctor_get(x_14, 4); +lean_inc(x_163); +x_164 = lean_ctor_get(x_163, 0); +lean_inc(x_164); +x_165 = 1; +x_166 = l_Lean_Language_SnapshotTask_bindIO___rarg(x_163, x_162, x_164, x_165, x_160); +if (lean_obj_tag(x_166) == 0) { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Language_instTypeNameSnapshotLeaf; -x_2 = l_Lean_Language_Lean_process_parseCmd___closed__1; -x_3 = l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Language_instInhabitedDynamicSnapshot___spec__1(x_1, x_2); -return x_3; +lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; +x_167 = lean_ctor_get(x_166, 1); +lean_inc(x_167); +lean_dec(x_166); +x_168 = lean_box(0); +x_169 = lean_io_promise_result(x_159); +if (lean_is_scalar(x_156)) { + x_170 = lean_alloc_ctor(0, 2, 0); +} else { + x_170 = x_156; } +lean_ctor_set(x_170, 0, x_168); +lean_ctor_set(x_170, 1, x_169); +x_171 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_171, 0, x_170); +if (lean_is_scalar(x_146)) { + x_172 = lean_alloc_ctor(0, 2, 0); +} else { + x_172 = x_146; } -static lean_object* _init_l_Lean_Language_Lean_process_parseCmd___closed__3() { -_start: +lean_ctor_set(x_172, 0, x_14); +lean_ctor_set(x_172, 1, x_171); +x_173 = lean_io_promise_resolve(x_172, x_4, x_167); +lean_dec(x_4); +if (lean_obj_tag(x_173) == 0) { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Language_Lean_process_parseCmd___closed__2; -x_2 = l_Lean_Language_SnapshotTask_pure___rarg(x_1); -return x_2; +lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; +x_174 = lean_ctor_get(x_173, 0); +lean_inc(x_174); +x_175 = lean_ctor_get(x_173, 1); +lean_inc(x_175); +if (lean_is_exclusive(x_173)) { + lean_ctor_release(x_173, 0); + lean_ctor_release(x_173, 1); + x_176 = x_173; +} else { + lean_dec_ref(x_173); + x_176 = lean_box(0); } +if (lean_is_scalar(x_176)) { + x_177 = lean_alloc_ctor(0, 2, 0); +} else { + x_177 = x_176; } -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -lean_object* x_7; lean_object* x_8; -x_7 = lean_ctor_get(x_5, 3); -lean_inc(x_7); -x_8 = lean_st_ref_get(x_7, x_6); -lean_dec(x_7); -if (lean_obj_tag(x_8) == 0) -{ -lean_object* x_9; uint8_t x_10; -x_9 = lean_ctor_get(x_8, 0); -lean_inc(x_9); -x_10 = lean_unbox(x_9); -lean_dec(x_9); -if (x_10 == 0) -{ -lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_11 = lean_ctor_get(x_8, 1); -lean_inc(x_11); -lean_dec(x_8); -x_12 = lean_box(0); -lean_inc(x_5); -x_13 = l_Lean_Language_Lean_process_parseCmd___lambda__8(x_2, x_3, x_5, x_4, x_1, x_12, x_5, x_11); -return x_13; +lean_ctor_set(x_177, 0, x_174); +lean_ctor_set(x_177, 1, x_175); +return x_177; } else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; -lean_dec(x_5); -lean_dec(x_1); -x_14 = lean_ctor_get(x_8, 1); -lean_inc(x_14); -lean_dec(x_8); -x_15 = l_Lean_Language_Lean_process_parseCmd___lambda__3___closed__1; -x_16 = lean_st_mk_ref(x_15, x_14); -if (lean_obj_tag(x_16) == 0) -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_16, 1); -lean_inc(x_18); -lean_dec(x_16); -x_19 = lean_box(0); -x_20 = l_Lean_Language_Lean_process_parseCmd___closed__1; -x_21 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_21, 0, x_20); -lean_ctor_set(x_21, 1, x_3); -x_22 = l_Lean_Language_SnapshotTask_pure___rarg(x_21); -x_23 = lean_box(0); -x_24 = l_Lean_Language_Lean_process_parseCmd___closed__3; -x_25 = lean_alloc_ctor(0, 6, 0); -lean_ctor_set(x_25, 0, x_20); -lean_ctor_set(x_25, 1, x_23); -lean_ctor_set(x_25, 2, x_2); -lean_ctor_set(x_25, 3, x_24); -lean_ctor_set(x_25, 4, x_22); -lean_ctor_set(x_25, 5, x_17); -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_26, 1, x_19); -x_27 = lean_io_promise_resolve(x_26, x_4, x_18); -lean_dec(x_4); -if (lean_obj_tag(x_27) == 0) -{ -uint8_t x_28; -x_28 = !lean_is_exclusive(x_27); -if (x_28 == 0) -{ -lean_object* x_29; lean_object* x_30; -x_29 = lean_ctor_get(x_27, 0); -lean_dec(x_29); -x_30 = lean_box(0); -lean_ctor_set(x_27, 0, x_30); -return x_27; +lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; +x_178 = lean_ctor_get(x_173, 0); +lean_inc(x_178); +x_179 = lean_ctor_get(x_173, 1); +lean_inc(x_179); +if (lean_is_exclusive(x_173)) { + lean_ctor_release(x_173, 0); + lean_ctor_release(x_173, 1); + x_180 = x_173; +} else { + lean_dec_ref(x_173); + x_180 = lean_box(0); } -else -{ -lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_31 = lean_ctor_get(x_27, 1); -lean_inc(x_31); -lean_dec(x_27); -x_32 = lean_box(0); -x_33 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_33, 0, x_32); -lean_ctor_set(x_33, 1, x_31); -return x_33; +if (lean_is_scalar(x_180)) { + x_181 = lean_alloc_ctor(1, 2, 0); +} else { + x_181 = x_180; } +lean_ctor_set(x_181, 0, x_178); +lean_ctor_set(x_181, 1, x_179); +return x_181; } -else -{ -uint8_t x_34; -x_34 = !lean_is_exclusive(x_27); -if (x_34 == 0) -{ -return x_27; } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_35 = lean_ctor_get(x_27, 0); -x_36 = lean_ctor_get(x_27, 1); -lean_inc(x_36); -lean_inc(x_35); -lean_dec(x_27); -x_37 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -return x_37; +lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; +lean_dec(x_159); +lean_dec(x_156); +lean_dec(x_146); +lean_dec(x_14); +lean_dec(x_4); +x_182 = lean_ctor_get(x_166, 0); +lean_inc(x_182); +x_183 = lean_ctor_get(x_166, 1); +lean_inc(x_183); +if (lean_is_exclusive(x_166)) { + lean_ctor_release(x_166, 0); + lean_ctor_release(x_166, 1); + x_184 = x_166; +} else { + lean_dec_ref(x_166); + x_184 = lean_box(0); } +if (lean_is_scalar(x_184)) { + x_185 = lean_alloc_ctor(1, 2, 0); +} else { + x_185 = x_184; +} +lean_ctor_set(x_185, 0, x_182); +lean_ctor_set(x_185, 1, x_183); +return x_185; } } else { -uint8_t x_38; +lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; +lean_dec(x_157); +lean_dec(x_156); +lean_dec(x_146); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_6); lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_38 = !lean_is_exclusive(x_16); -if (x_38 == 0) -{ -return x_16; +x_186 = lean_ctor_get(x_158, 0); +lean_inc(x_186); +x_187 = lean_ctor_get(x_158, 1); +lean_inc(x_187); +if (lean_is_exclusive(x_158)) { + lean_ctor_release(x_158, 0); + lean_ctor_release(x_158, 1); + x_188 = x_158; +} else { + lean_dec_ref(x_158); + x_188 = lean_box(0); +} +if (lean_is_scalar(x_188)) { + x_189 = lean_alloc_ctor(1, 2, 0); +} else { + x_189 = x_188; +} +lean_ctor_set(x_189, 0, x_186); +lean_ctor_set(x_189, 1, x_187); +return x_189; } -else -{ -lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_39 = lean_ctor_get(x_16, 0); -x_40 = lean_ctor_get(x_16, 1); -lean_inc(x_40); -lean_inc(x_39); -lean_dec(x_16); -x_41 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_41, 0, x_39); -lean_ctor_set(x_41, 1, x_40); -return x_41; } } } } else { -uint8_t x_42; -lean_dec(x_5); +uint8_t x_190; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_6); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_42 = !lean_is_exclusive(x_8); -if (x_42 == 0) +x_190 = !lean_is_exclusive(x_16); +if (x_190 == 0) { -return x_8; +return x_16; } else -{ -lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_43 = lean_ctor_get(x_8, 0); -x_44 = lean_ctor_get(x_8, 1); -lean_inc(x_44); -lean_inc(x_43); -lean_dec(x_8); -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_191; lean_object* x_192; lean_object* x_193; +x_191 = lean_ctor_get(x_16, 0); +x_192 = lean_ctor_get(x_16, 1); +lean_inc(x_192); +lean_inc(x_191); +lean_dec(x_16); +x_193 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_193, 0, x_191); +lean_ctor_set(x_193, 1, x_192); +return x_193; +} +} } } } @@ -7633,56 +8085,100 @@ lean_dec(x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___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_17; lean_object* x_18; -x_17 = lean_unbox(x_12); +uint8_t x_16; lean_object* x_17; +x_16 = lean_unbox(x_12); lean_dec(x_12); -x_18 = l_Lean_Language_Lean_process_parseCmd___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_17, x_13, x_14, x_15, x_16); -lean_dec(x_15); +x_17 = l_Lean_Language_Lean_process_parseCmd___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_16, x_13, x_14, x_15); lean_dec(x_8); lean_dec(x_2); -return x_18; +return x_17; } } -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_13; -x_13 = l_Lean_Language_Lean_process_parseCmd___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_11); -lean_dec(x_10); +lean_object* x_12; +x_12 = l_Lean_Language_Lean_process_parseCmd___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_4); lean_dec(x_2); -return x_13; +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +uint8_t x_14; lean_object* x_15; +x_14 = lean_unbox(x_1); +lean_dec(x_1); +x_15 = l_Lean_Language_Lean_process_parseCmd___lambda__4(x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_12); +lean_dec(x_11); +return x_15; +} +} +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___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) { +_start: +{ +uint8_t x_14; lean_object* x_15; +x_14 = lean_unbox(x_2); +lean_dec(x_2); +x_15 = l_Lean_Language_Lean_process_parseCmd___lambda__5(x_1, x_14, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_12); +lean_dec(x_11); +return x_15; } } -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__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_Language_Lean_process_parseCmd___lambda__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; -x_6 = l_Lean_Language_Lean_process_parseCmd___lambda__4(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Lean_Language_Lean_process_parseCmd___lambda__6(x_1, x_2, x_3, x_4, x_5); lean_dec(x_3); lean_dec(x_1); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___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_9; -x_9 = l_Lean_Language_Lean_process_parseCmd___lambda__7(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_6); +uint8_t x_8; lean_object* x_9; +x_8 = lean_unbox(x_4); +lean_dec(x_4); +x_9 = l_Lean_Language_Lean_process_parseCmd___lambda__7(x_1, x_2, x_3, x_8, x_5, x_6, x_7); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___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_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___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_9; -x_9 = l_Lean_Language_Lean_process_parseCmd___lambda__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_6); +uint8_t x_8; lean_object* x_9; +x_8 = lean_unbox(x_3); +lean_dec(x_3); +x_9 = l_Lean_Language_Lean_process_parseCmd___lambda__8(x_1, x_2, x_8, x_4, x_5, x_6, x_7); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___lambda__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +uint8_t x_10; lean_object* x_11; +x_10 = lean_unbox(x_4); +lean_dec(x_4); +x_11 = l_Lean_Language_Lean_process_parseCmd___lambda__9(x_1, x_2, x_3, x_10, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_7); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_parseCmd___boxed(lean_object* x_1, 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_5); +lean_dec(x_5); +x_9 = l_Lean_Language_Lean_process_parseCmd(x_1, x_2, x_3, x_4, x_8, x_6, x_7); return x_9; } } @@ -7861,32 +8357,7 @@ x_6 = lean_apply_3(x_1, x_2, x_5, x_4); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_processHeader___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; uint8_t x_8; -x_7 = l_Lean_Language_Lean_process_parseCmd(x_1, x_2, x_3, x_4, x_5, x_6); -x_8 = !lean_is_exclusive(x_7); -if (x_8 == 0) -{ -return x_7; -} -else -{ -lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_9 = lean_ctor_get(x_7, 0); -x_10 = lean_ctor_get(x_7, 1); -lean_inc(x_10); -lean_inc(x_9); -lean_dec(x_7); -x_11 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_11, 0, x_9); -lean_ctor_set(x_11, 1, x_10); -return x_11; -} -} -} -static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__4___closed__1() { +static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__3___closed__1() { _start: { lean_object* x_1; @@ -7894,7 +8365,7 @@ x_1 = l_Lean_maxRecDepth; return x_1; } } -static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__4___closed__2() { +static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__3___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -7913,7 +8384,7 @@ lean_ctor_set(x_3, 8, x_2); return x_3; } } -static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__4___closed__3() { +static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__3___closed__3() { _start: { lean_object* x_1; @@ -7921,21 +8392,21 @@ x_1 = lean_mk_string_unchecked("_import", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__4___closed__4() { +static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__3___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__3; +x_2 = l_Lean_Language_Lean_process_processHeader___lambda__3___closed__3; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__4___closed__5() { +static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__3___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__4; +x_1 = l_Lean_Language_Lean_process_processHeader___lambda__3___closed__4; x_2 = lean_unsigned_to_nat(1u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -7943,7 +8414,7 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__4___closed__6() { +static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__3___closed__6() { _start: { lean_object* x_1; @@ -7951,17 +8422,17 @@ x_1 = lean_mk_string_unchecked("header", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__4___closed__7() { +static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__3___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__6; +x_2 = l_Lean_Language_Lean_process_processHeader___lambda__3___closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__4___closed__8() { +static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__3___closed__8() { _start: { lean_object* x_1; @@ -7969,30 +8440,30 @@ x_1 = lean_mk_string_unchecked("processHeader", 13, 13); return x_1; } } -static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__4___closed__9() { +static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__3___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Language_Lean_initFn____x40_Lean_Language_Lean___hyg_10____closed__6; x_2 = l_Lean_Language_Lean_initFn____x40_Lean_Language_Lean___hyg_10____closed__7; x_3 = l_Lean_Language_Lean_process_doElab___lambda__4___closed__1; -x_4 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__8; +x_4 = l_Lean_Language_Lean_process_processHeader___lambda__3___closed__8; x_5 = l_Lean_Name_mkStr5(x_1, x_2, x_1, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__4___closed__10() { +static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__3___closed__10() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__9; +x_1 = l_Lean_Language_Lean_process_processHeader___lambda__3___closed__9; x_2 = 1; x_3 = l___private_Lean_Language_Lean_0__Lean_Language_Lean_withHeaderExceptions___rarg___closed__12; x_4 = l_Lean_Name_toString(x_1, x_2, x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_processHeader___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_Language_Lean_process_processHeader___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; @@ -8025,14 +8496,14 @@ x_22 = lean_ctor_get(x_16, 1); lean_dec(x_22); x_23 = lean_ctor_get(x_16, 0); lean_dec(x_23); -x_24 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__1; +x_24 = l_Lean_Language_Lean_process_processHeader___lambda__3___closed__1; x_25 = l_Lean_Option_get___at_Lean_profiler_threshold_getSecs___spec__1(x_14, x_24); lean_dec(x_14); x_26 = lean_ctor_get(x_4, 2); x_27 = lean_box(0); -x_28 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__2; +x_28 = l_Lean_Language_Lean_process_processHeader___lambda__3___closed__2; x_29 = lean_box(0); -x_30 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__5; +x_30 = l_Lean_Language_Lean_process_processHeader___lambda__3___closed__5; lean_inc(x_26); lean_inc(x_2); x_31 = lean_alloc_ctor(0, 7, 0); @@ -8045,7 +8516,7 @@ lean_ctor_set(x_31, 5, x_27); lean_ctor_set(x_31, 6, x_30); x_32 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_32, 0, x_31); -x_33 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__7; +x_33 = l_Lean_Language_Lean_process_processHeader___lambda__3___closed__7; lean_inc(x_5); x_34 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_34, 0, x_33); @@ -8089,7 +8560,7 @@ x_51 = lean_io_promise_new(x_15); x_52 = !lean_is_exclusive(x_51); 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; lean_object* x_62; uint8_t x_63; +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_53 = lean_ctor_get(x_51, 0); x_54 = lean_ctor_get(x_51, 1); x_55 = lean_runtime_mark_persistent(x_6); @@ -8098,452 +8569,425 @@ x_57 = lean_runtime_mark_persistent(x_7); x_58 = lean_box(0); lean_inc(x_53); lean_inc(x_56); -x_59 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_processHeader___lambda__3), 6, 5); -lean_closure_set(x_59, 0, x_58); -lean_closure_set(x_59, 1, x_55); -lean_closure_set(x_59, 2, x_56); -lean_closure_set(x_59, 3, x_53); -lean_closure_set(x_59, 4, x_57); -x_60 = lean_alloc_closure((void*)(l_EIO_toBaseIO___rarg), 2, 1); -lean_closure_set(x_60, 0, x_59); -x_61 = l_Task_Priority_default; -x_62 = lean_io_as_task(x_60, x_61, x_54); -x_63 = !lean_is_exclusive(x_62); -if (x_63 == 0) +x_59 = l_Lean_Language_Lean_process_parseCmd(x_58, x_55, x_56, x_53, x_47, x_57, x_54); +x_60 = !lean_is_exclusive(x_59); +if (x_60 == 0) { -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; -x_64 = lean_ctor_get(x_62, 0); +lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; uint8_t x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; +x_61 = lean_ctor_get(x_59, 0); +lean_dec(x_61); +x_62 = lean_ctor_get(x_56, 6); +lean_inc(x_62); +x_63 = lean_ctor_get(x_62, 1); +lean_inc(x_63); +lean_dec(x_62); +x_64 = lean_ctor_get(x_63, 2); +lean_inc(x_64); +x_65 = lean_unsigned_to_nat(0u); +x_66 = lean_nat_dec_lt(x_65, x_64); lean_dec(x_64); -x_65 = lean_ctor_get(x_56, 6); -lean_inc(x_65); -x_66 = lean_ctor_get(x_65, 1); -lean_inc(x_66); -lean_dec(x_65); -x_67 = lean_ctor_get(x_66, 2); -lean_inc(x_67); -x_68 = lean_unsigned_to_nat(0u); -x_69 = lean_nat_dec_lt(x_68, x_67); -lean_dec(x_67); -x_70 = lean_io_promise_result(x_53); -lean_ctor_set(x_51, 1, x_70); +x_67 = lean_io_promise_result(x_53); +lean_ctor_set(x_51, 1, x_67); lean_ctor_set(x_51, 0, x_58); -x_71 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_71, 0, x_56); -lean_ctor_set(x_71, 1, x_51); +x_68 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_68, 0, x_56); +lean_ctor_set(x_68, 1, x_51); +x_69 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_69, 0, x_68); +if (x_66 == 0) +{ +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_dec(x_63); +x_70 = l_Lean_Elab_instInhabitedInfoTree; +x_71 = l_outOfBounds___rarg(x_70); x_72 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_72, 0, x_71); -if (x_69 == 0) -{ -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_dec(x_66); -x_73 = l_Lean_Elab_instInhabitedInfoTree; -x_74 = l_outOfBounds___rarg(x_73); -x_75 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_75, 0, x_74); -x_76 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__10; -x_77 = 0; -x_78 = lean_alloc_ctor(0, 3, 1); -lean_ctor_set(x_78, 0, x_76); -lean_ctor_set(x_78, 1, x_8); -lean_ctor_set(x_78, 2, x_75); -lean_ctor_set_uint8(x_78, sizeof(void*)*3, 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_72); -lean_ctor_set(x_62, 0, x_79); -return x_62; +x_73 = l_Lean_Language_Lean_process_processHeader___lambda__3___closed__10; +x_74 = 0; +x_75 = lean_alloc_ctor(0, 3, 1); +lean_ctor_set(x_75, 0, x_73); +lean_ctor_set(x_75, 1, x_8); +lean_ctor_set(x_75, 2, x_72); +lean_ctor_set_uint8(x_75, sizeof(void*)*3, x_74); +x_76 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_76, 0, x_75); +lean_ctor_set(x_76, 1, x_69); +lean_ctor_set(x_59, 0, x_76); +return x_59; } 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; -x_80 = l_Lean_Elab_instInhabitedInfoTree; -x_81 = l_Lean_PersistentArray_get_x21___rarg(x_80, x_66, x_68); -x_82 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_82, 0, x_81); -x_83 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__10; -x_84 = 0; -x_85 = lean_alloc_ctor(0, 3, 1); -lean_ctor_set(x_85, 0, x_83); -lean_ctor_set(x_85, 1, x_8); -lean_ctor_set(x_85, 2, x_82); -lean_ctor_set_uint8(x_85, sizeof(void*)*3, x_84); -x_86 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_86, 0, x_85); -lean_ctor_set(x_86, 1, x_72); -lean_ctor_set(x_62, 0, x_86); -return x_62; +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_Lean_Elab_instInhabitedInfoTree; +x_78 = l_Lean_PersistentArray_get_x21___rarg(x_77, x_63, x_65); +x_79 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_79, 0, x_78); +x_80 = l_Lean_Language_Lean_process_processHeader___lambda__3___closed__10; +x_81 = 0; +x_82 = lean_alloc_ctor(0, 3, 1); +lean_ctor_set(x_82, 0, x_80); +lean_ctor_set(x_82, 1, x_8); +lean_ctor_set(x_82, 2, x_79); +lean_ctor_set_uint8(x_82, sizeof(void*)*3, 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_69); +lean_ctor_set(x_59, 0, x_83); +return x_59; } } else { -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; -x_87 = lean_ctor_get(x_62, 1); +lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; uint8_t x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; +x_84 = lean_ctor_get(x_59, 1); +lean_inc(x_84); +lean_dec(x_59); +x_85 = lean_ctor_get(x_56, 6); +lean_inc(x_85); +x_86 = lean_ctor_get(x_85, 1); +lean_inc(x_86); +lean_dec(x_85); +x_87 = lean_ctor_get(x_86, 2); lean_inc(x_87); -lean_dec(x_62); -x_88 = lean_ctor_get(x_56, 6); -lean_inc(x_88); -x_89 = lean_ctor_get(x_88, 1); -lean_inc(x_89); -lean_dec(x_88); -x_90 = lean_ctor_get(x_89, 2); -lean_inc(x_90); -x_91 = lean_unsigned_to_nat(0u); -x_92 = lean_nat_dec_lt(x_91, x_90); -lean_dec(x_90); -x_93 = lean_io_promise_result(x_53); -lean_ctor_set(x_51, 1, x_93); +x_88 = lean_unsigned_to_nat(0u); +x_89 = lean_nat_dec_lt(x_88, x_87); +lean_dec(x_87); +x_90 = lean_io_promise_result(x_53); +lean_ctor_set(x_51, 1, x_90); lean_ctor_set(x_51, 0, x_58); -x_94 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_94, 0, x_56); -lean_ctor_set(x_94, 1, x_51); +x_91 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_91, 0, x_56); +lean_ctor_set(x_91, 1, x_51); +x_92 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_92, 0, x_91); +if (x_89 == 0) +{ +lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; uint8_t x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; +lean_dec(x_86); +x_93 = l_Lean_Elab_instInhabitedInfoTree; +x_94 = l_outOfBounds___rarg(x_93); x_95 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_95, 0, x_94); -if (x_92 == 0) -{ -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_dec(x_89); -x_96 = l_Lean_Elab_instInhabitedInfoTree; -x_97 = l_outOfBounds___rarg(x_96); -x_98 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_98, 0, x_97); -x_99 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__10; -x_100 = 0; -x_101 = lean_alloc_ctor(0, 3, 1); -lean_ctor_set(x_101, 0, x_99); -lean_ctor_set(x_101, 1, x_8); -lean_ctor_set(x_101, 2, x_98); -lean_ctor_set_uint8(x_101, sizeof(void*)*3, x_100); -x_102 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_102, 0, x_101); -lean_ctor_set(x_102, 1, x_95); -x_103 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_103, 0, x_102); -lean_ctor_set(x_103, 1, x_87); -return x_103; +x_96 = l_Lean_Language_Lean_process_processHeader___lambda__3___closed__10; +x_97 = 0; +x_98 = lean_alloc_ctor(0, 3, 1); +lean_ctor_set(x_98, 0, x_96); +lean_ctor_set(x_98, 1, x_8); +lean_ctor_set(x_98, 2, x_95); +lean_ctor_set_uint8(x_98, sizeof(void*)*3, 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_92); +x_100 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_100, 0, x_99); +lean_ctor_set(x_100, 1, x_84); +return x_100; } else { -lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; uint8_t x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; -x_104 = l_Lean_Elab_instInhabitedInfoTree; -x_105 = l_Lean_PersistentArray_get_x21___rarg(x_104, x_89, x_91); -x_106 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_106, 0, x_105); -x_107 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__10; -x_108 = 0; -x_109 = lean_alloc_ctor(0, 3, 1); -lean_ctor_set(x_109, 0, x_107); -lean_ctor_set(x_109, 1, x_8); -lean_ctor_set(x_109, 2, x_106); -lean_ctor_set_uint8(x_109, sizeof(void*)*3, x_108); -x_110 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_110, 0, x_109); -lean_ctor_set(x_110, 1, x_95); -x_111 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_111, 0, x_110); -lean_ctor_set(x_111, 1, x_87); -return x_111; +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_object* x_108; +x_101 = l_Lean_Elab_instInhabitedInfoTree; +x_102 = l_Lean_PersistentArray_get_x21___rarg(x_101, x_86, x_88); +x_103 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_103, 0, x_102); +x_104 = l_Lean_Language_Lean_process_processHeader___lambda__3___closed__10; +x_105 = 0; +x_106 = lean_alloc_ctor(0, 3, 1); +lean_ctor_set(x_106, 0, x_104); +lean_ctor_set(x_106, 1, x_8); +lean_ctor_set(x_106, 2, x_103); +lean_ctor_set_uint8(x_106, sizeof(void*)*3, x_105); +x_107 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_107, 0, x_106); +lean_ctor_set(x_107, 1, x_92); +x_108 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_108, 0, x_107); +lean_ctor_set(x_108, 1, x_84); +return x_108; } } } 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; uint8_t x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; -x_112 = lean_ctor_get(x_51, 0); -x_113 = lean_ctor_get(x_51, 1); -lean_inc(x_113); -lean_inc(x_112); +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; uint8_t x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; +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_dec(x_51); -x_114 = lean_runtime_mark_persistent(x_6); -x_115 = lean_runtime_mark_persistent(x_16); -x_116 = lean_runtime_mark_persistent(x_7); -x_117 = lean_box(0); +x_111 = lean_runtime_mark_persistent(x_6); +x_112 = lean_runtime_mark_persistent(x_16); +x_113 = lean_runtime_mark_persistent(x_7); +x_114 = lean_box(0); +lean_inc(x_109); lean_inc(x_112); -lean_inc(x_115); -x_118 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_processHeader___lambda__3), 6, 5); -lean_closure_set(x_118, 0, x_117); -lean_closure_set(x_118, 1, x_114); -lean_closure_set(x_118, 2, x_115); -lean_closure_set(x_118, 3, x_112); -lean_closure_set(x_118, 4, x_116); -x_119 = lean_alloc_closure((void*)(l_EIO_toBaseIO___rarg), 2, 1); -lean_closure_set(x_119, 0, x_118); -x_120 = l_Task_Priority_default; -x_121 = lean_io_as_task(x_119, x_120, x_113); -x_122 = lean_ctor_get(x_121, 1); -lean_inc(x_122); -if (lean_is_exclusive(x_121)) { - lean_ctor_release(x_121, 0); - lean_ctor_release(x_121, 1); - x_123 = x_121; -} else { - lean_dec_ref(x_121); - x_123 = lean_box(0); -} -x_124 = lean_ctor_get(x_115, 6); -lean_inc(x_124); -x_125 = lean_ctor_get(x_124, 1); -lean_inc(x_125); -lean_dec(x_124); -x_126 = lean_ctor_get(x_125, 2); -lean_inc(x_126); -x_127 = lean_unsigned_to_nat(0u); -x_128 = lean_nat_dec_lt(x_127, x_126); -lean_dec(x_126); -x_129 = lean_io_promise_result(x_112); -x_130 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_130, 0, x_117); -lean_ctor_set(x_130, 1, x_129); -x_131 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_131, 0, x_115); -lean_ctor_set(x_131, 1, x_130); -x_132 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_132, 0, x_131); -if (x_128 == 0) -{ -lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; uint8_t x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; -lean_dec(x_125); -x_133 = l_Lean_Elab_instInhabitedInfoTree; -x_134 = l_outOfBounds___rarg(x_133); -x_135 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_135, 0, x_134); -x_136 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__10; -x_137 = 0; -x_138 = lean_alloc_ctor(0, 3, 1); -lean_ctor_set(x_138, 0, x_136); -lean_ctor_set(x_138, 1, x_8); -lean_ctor_set(x_138, 2, x_135); -lean_ctor_set_uint8(x_138, sizeof(void*)*3, 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_132); -if (lean_is_scalar(x_123)) { - x_140 = lean_alloc_ctor(0, 2, 0); +x_115 = l_Lean_Language_Lean_process_parseCmd(x_114, x_111, x_112, x_109, x_47, x_113, x_110); +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 { - x_140 = x_123; -} -lean_ctor_set(x_140, 0, x_139); -lean_ctor_set(x_140, 1, x_122); -return x_140; + lean_dec_ref(x_115); + x_117 = lean_box(0); } -else +x_118 = lean_ctor_get(x_112, 6); +lean_inc(x_118); +x_119 = lean_ctor_get(x_118, 1); +lean_inc(x_119); +lean_dec(x_118); +x_120 = lean_ctor_get(x_119, 2); +lean_inc(x_120); +x_121 = lean_unsigned_to_nat(0u); +x_122 = lean_nat_dec_lt(x_121, x_120); +lean_dec(x_120); +x_123 = lean_io_promise_result(x_109); +x_124 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_124, 0, x_114); +lean_ctor_set(x_124, 1, x_123); +x_125 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_125, 0, x_112); +lean_ctor_set(x_125, 1, x_124); +x_126 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_126, 0, x_125); +if (x_122 == 0) { -lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; uint8_t x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; -x_141 = l_Lean_Elab_instInhabitedInfoTree; -x_142 = l_Lean_PersistentArray_get_x21___rarg(x_141, x_125, x_127); -x_143 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_143, 0, x_142); -x_144 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__10; -x_145 = 0; -x_146 = lean_alloc_ctor(0, 3, 1); -lean_ctor_set(x_146, 0, x_144); -lean_ctor_set(x_146, 1, x_8); -lean_ctor_set(x_146, 2, x_143); -lean_ctor_set_uint8(x_146, sizeof(void*)*3, 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_132); -if (lean_is_scalar(x_123)) { - x_148 = lean_alloc_ctor(0, 2, 0); +lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; uint8_t x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; +lean_dec(x_119); +x_127 = l_Lean_Elab_instInhabitedInfoTree; +x_128 = l_outOfBounds___rarg(x_127); +x_129 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_129, 0, x_128); +x_130 = l_Lean_Language_Lean_process_processHeader___lambda__3___closed__10; +x_131 = 0; +x_132 = lean_alloc_ctor(0, 3, 1); +lean_ctor_set(x_132, 0, x_130); +lean_ctor_set(x_132, 1, x_8); +lean_ctor_set(x_132, 2, x_129); +lean_ctor_set_uint8(x_132, sizeof(void*)*3, x_131); +x_133 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_133, 0, x_132); +lean_ctor_set(x_133, 1, x_126); +if (lean_is_scalar(x_117)) { + x_134 = lean_alloc_ctor(0, 2, 0); +} else { + x_134 = x_117; +} +lean_ctor_set(x_134, 0, x_133); +lean_ctor_set(x_134, 1, x_116); +return x_134; +} +else +{ +lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; uint8_t x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; +x_135 = l_Lean_Elab_instInhabitedInfoTree; +x_136 = l_Lean_PersistentArray_get_x21___rarg(x_135, x_119, x_121); +x_137 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_137, 0, x_136); +x_138 = l_Lean_Language_Lean_process_processHeader___lambda__3___closed__10; +x_139 = 0; +x_140 = lean_alloc_ctor(0, 3, 1); +lean_ctor_set(x_140, 0, x_138); +lean_ctor_set(x_140, 1, x_8); +lean_ctor_set(x_140, 2, x_137); +lean_ctor_set_uint8(x_140, sizeof(void*)*3, x_139); +x_141 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_141, 0, x_140); +lean_ctor_set(x_141, 1, x_126); +if (lean_is_scalar(x_117)) { + x_142 = lean_alloc_ctor(0, 2, 0); } else { - x_148 = x_123; + x_142 = x_117; } -lean_ctor_set(x_148, 0, x_147); -lean_ctor_set(x_148, 1, x_122); -return x_148; +lean_ctor_set(x_142, 0, x_141); +lean_ctor_set(x_142, 1, x_116); +return x_142; } } } else { -lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; 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; 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; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; uint8_t x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; -x_149 = lean_ctor_get(x_16, 2); -x_150 = lean_ctor_get(x_16, 5); -lean_inc(x_150); -lean_inc(x_149); +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; uint8_t 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; uint8_t x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; +x_143 = lean_ctor_get(x_16, 2); +x_144 = lean_ctor_get(x_16, 5); +lean_inc(x_144); +lean_inc(x_143); lean_dec(x_16); -x_151 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__1; -x_152 = l_Lean_Option_get___at_Lean_profiler_threshold_getSecs___spec__1(x_14, x_151); +x_145 = l_Lean_Language_Lean_process_processHeader___lambda__3___closed__1; +x_146 = l_Lean_Option_get___at_Lean_profiler_threshold_getSecs___spec__1(x_14, x_145); lean_dec(x_14); -x_153 = lean_ctor_get(x_4, 2); -x_154 = lean_box(0); -x_155 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__2; -x_156 = lean_box(0); -x_157 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__5; -lean_inc(x_153); +x_147 = lean_ctor_get(x_4, 2); +x_148 = lean_box(0); +x_149 = l_Lean_Language_Lean_process_processHeader___lambda__3___closed__2; +x_150 = lean_box(0); +x_151 = l_Lean_Language_Lean_process_processHeader___lambda__3___closed__5; +lean_inc(x_147); lean_inc(x_2); -x_158 = lean_alloc_ctor(0, 7, 0); -lean_ctor_set(x_158, 0, x_2); -lean_ctor_set(x_158, 1, x_153); -lean_ctor_set(x_158, 2, x_155); -lean_ctor_set(x_158, 3, x_154); -lean_ctor_set(x_158, 4, x_156); -lean_ctor_set(x_158, 5, x_154); -lean_ctor_set(x_158, 6, x_157); -x_159 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_159, 0, x_158); -x_160 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__7; +x_152 = lean_alloc_ctor(0, 7, 0); +lean_ctor_set(x_152, 0, x_2); +lean_ctor_set(x_152, 1, x_147); +lean_ctor_set(x_152, 2, x_149); +lean_ctor_set(x_152, 3, x_148); +lean_ctor_set(x_152, 4, x_150); +lean_ctor_set(x_152, 5, x_148); +lean_ctor_set(x_152, 6, x_151); +x_153 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_153, 0, x_152); +x_154 = l_Lean_Language_Lean_process_processHeader___lambda__3___closed__7; lean_inc(x_5); -x_161 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_161, 0, x_160); -lean_ctor_set(x_161, 1, x_5); -x_162 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_162, 0, x_161); -x_163 = lean_unsigned_to_nat(1u); -x_164 = l_Lean_Syntax_getArg(x_5, x_163); +x_155 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_155, 0, x_154); +lean_ctor_set(x_155, 1, x_5); +x_156 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_156, 0, x_155); +x_157 = lean_unsigned_to_nat(1u); +x_158 = l_Lean_Syntax_getArg(x_5, x_157); lean_dec(x_5); -x_165 = l_Lean_Syntax_getArgs(x_164); -lean_dec(x_164); -x_166 = lean_array_to_list(x_165); -x_167 = l_List_mapTR_loop___at_Lean_Language_Lean_process_processHeader___spec__1(x_166, x_154); -x_168 = l_List_toPArray_x27___rarg(x_167); -x_169 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_169, 0, x_162); -lean_ctor_set(x_169, 1, x_168); -x_170 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_170, 0, x_159); -lean_ctor_set(x_170, 1, x_169); -x_171 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_171, 0, x_170); -lean_ctor_set(x_171, 1, x_154); -x_172 = lean_array_mk(x_171); -x_173 = l_Array_toPArray_x27___rarg(x_172); -lean_dec(x_172); -x_174 = 1; -x_175 = l_Lean_Language_Lean_process_doElab___closed__4; -x_176 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_176, 0, x_175); -lean_ctor_set(x_176, 1, x_173); -lean_ctor_set_uint8(x_176, sizeof(void*)*2, x_174); -x_177 = l_Lean_Language_Lean_process_doElab___lambda__3___closed__5; -x_178 = lean_alloc_ctor(0, 8, 0); -lean_ctor_set(x_178, 0, x_2); -lean_ctor_set(x_178, 1, x_3); -lean_ctor_set(x_178, 2, x_149); -lean_ctor_set(x_178, 3, x_177); -lean_ctor_set(x_178, 4, x_152); -lean_ctor_set(x_178, 5, x_150); -lean_ctor_set(x_178, 6, x_176); -lean_ctor_set(x_178, 7, x_9); -x_179 = lean_io_promise_new(x_15); -x_180 = lean_ctor_get(x_179, 0); -lean_inc(x_180); -x_181 = lean_ctor_get(x_179, 1); -lean_inc(x_181); -if (lean_is_exclusive(x_179)) { - lean_ctor_release(x_179, 0); - lean_ctor_release(x_179, 1); - x_182 = x_179; +x_159 = l_Lean_Syntax_getArgs(x_158); +lean_dec(x_158); +x_160 = lean_array_to_list(x_159); +x_161 = l_List_mapTR_loop___at_Lean_Language_Lean_process_processHeader___spec__1(x_160, x_148); +x_162 = l_List_toPArray_x27___rarg(x_161); +x_163 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_163, 0, x_156); +lean_ctor_set(x_163, 1, x_162); +x_164 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_164, 0, x_153); +lean_ctor_set(x_164, 1, x_163); +x_165 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_165, 0, x_164); +lean_ctor_set(x_165, 1, x_148); +x_166 = lean_array_mk(x_165); +x_167 = l_Array_toPArray_x27___rarg(x_166); +lean_dec(x_166); +x_168 = 1; +x_169 = l_Lean_Language_Lean_process_doElab___closed__4; +x_170 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_170, 0, x_169); +lean_ctor_set(x_170, 1, x_167); +lean_ctor_set_uint8(x_170, sizeof(void*)*2, x_168); +x_171 = l_Lean_Language_Lean_process_doElab___lambda__3___closed__5; +x_172 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_172, 0, x_2); +lean_ctor_set(x_172, 1, x_3); +lean_ctor_set(x_172, 2, x_143); +lean_ctor_set(x_172, 3, x_171); +lean_ctor_set(x_172, 4, x_146); +lean_ctor_set(x_172, 5, x_144); +lean_ctor_set(x_172, 6, x_170); +lean_ctor_set(x_172, 7, x_9); +x_173 = lean_io_promise_new(x_15); +x_174 = lean_ctor_get(x_173, 0); +lean_inc(x_174); +x_175 = lean_ctor_get(x_173, 1); +lean_inc(x_175); +if (lean_is_exclusive(x_173)) { + lean_ctor_release(x_173, 0); + lean_ctor_release(x_173, 1); + x_176 = x_173; } else { - lean_dec_ref(x_179); - x_182 = lean_box(0); + lean_dec_ref(x_173); + x_176 = lean_box(0); } -x_183 = lean_runtime_mark_persistent(x_6); -x_184 = lean_runtime_mark_persistent(x_178); -x_185 = lean_runtime_mark_persistent(x_7); -x_186 = lean_box(0); -lean_inc(x_180); +x_177 = lean_runtime_mark_persistent(x_6); +x_178 = lean_runtime_mark_persistent(x_172); +x_179 = lean_runtime_mark_persistent(x_7); +x_180 = lean_box(0); +lean_inc(x_174); +lean_inc(x_178); +x_181 = l_Lean_Language_Lean_process_parseCmd(x_180, x_177, x_178, x_174, x_168, x_179, x_175); +x_182 = lean_ctor_get(x_181, 1); +lean_inc(x_182); +if (lean_is_exclusive(x_181)) { + lean_ctor_release(x_181, 0); + lean_ctor_release(x_181, 1); + x_183 = x_181; +} else { + lean_dec_ref(x_181); + x_183 = lean_box(0); +} +x_184 = lean_ctor_get(x_178, 6); lean_inc(x_184); -x_187 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_processHeader___lambda__3), 6, 5); -lean_closure_set(x_187, 0, x_186); -lean_closure_set(x_187, 1, x_183); -lean_closure_set(x_187, 2, x_184); -lean_closure_set(x_187, 3, x_180); -lean_closure_set(x_187, 4, x_185); -x_188 = lean_alloc_closure((void*)(l_EIO_toBaseIO___rarg), 2, 1); -lean_closure_set(x_188, 0, x_187); -x_189 = l_Task_Priority_default; -x_190 = lean_io_as_task(x_188, x_189, x_181); -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_185 = lean_ctor_get(x_184, 1); +lean_inc(x_185); +lean_dec(x_184); +x_186 = lean_ctor_get(x_185, 2); +lean_inc(x_186); +x_187 = lean_unsigned_to_nat(0u); +x_188 = lean_nat_dec_lt(x_187, x_186); +lean_dec(x_186); +x_189 = lean_io_promise_result(x_174); +if (lean_is_scalar(x_176)) { + x_190 = lean_alloc_ctor(0, 2, 0); } else { - lean_dec_ref(x_190); - x_192 = lean_box(0); + x_190 = x_176; } -x_193 = lean_ctor_get(x_184, 6); -lean_inc(x_193); -x_194 = lean_ctor_get(x_193, 1); -lean_inc(x_194); -lean_dec(x_193); -x_195 = lean_ctor_get(x_194, 2); -lean_inc(x_195); -x_196 = lean_unsigned_to_nat(0u); -x_197 = lean_nat_dec_lt(x_196, x_195); -lean_dec(x_195); -x_198 = lean_io_promise_result(x_180); -if (lean_is_scalar(x_182)) { - x_199 = lean_alloc_ctor(0, 2, 0); -} else { - x_199 = x_182; -} -lean_ctor_set(x_199, 0, x_186); -lean_ctor_set(x_199, 1, x_198); -x_200 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_200, 0, x_184); -lean_ctor_set(x_200, 1, x_199); -x_201 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_201, 0, x_200); -if (x_197 == 0) -{ -lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; uint8_t x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; -lean_dec(x_194); -x_202 = l_Lean_Elab_instInhabitedInfoTree; -x_203 = l_outOfBounds___rarg(x_202); -x_204 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_204, 0, x_203); -x_205 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__10; -x_206 = 0; -x_207 = lean_alloc_ctor(0, 3, 1); -lean_ctor_set(x_207, 0, x_205); -lean_ctor_set(x_207, 1, x_8); -lean_ctor_set(x_207, 2, x_204); -lean_ctor_set_uint8(x_207, sizeof(void*)*3, x_206); -x_208 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_208, 0, x_207); -lean_ctor_set(x_208, 1, x_201); -if (lean_is_scalar(x_192)) { - x_209 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_190, 0, x_180); +lean_ctor_set(x_190, 1, x_189); +x_191 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_191, 0, x_178); +lean_ctor_set(x_191, 1, x_190); +x_192 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_192, 0, x_191); +if (x_188 == 0) +{ +lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; uint8_t x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; +lean_dec(x_185); +x_193 = l_Lean_Elab_instInhabitedInfoTree; +x_194 = l_outOfBounds___rarg(x_193); +x_195 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_195, 0, x_194); +x_196 = l_Lean_Language_Lean_process_processHeader___lambda__3___closed__10; +x_197 = 0; +x_198 = lean_alloc_ctor(0, 3, 1); +lean_ctor_set(x_198, 0, x_196); +lean_ctor_set(x_198, 1, x_8); +lean_ctor_set(x_198, 2, x_195); +lean_ctor_set_uint8(x_198, sizeof(void*)*3, x_197); +x_199 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_199, 0, x_198); +lean_ctor_set(x_199, 1, x_192); +if (lean_is_scalar(x_183)) { + x_200 = lean_alloc_ctor(0, 2, 0); } else { - x_209 = x_192; + x_200 = x_183; } -lean_ctor_set(x_209, 0, x_208); -lean_ctor_set(x_209, 1, x_191); -return x_209; +lean_ctor_set(x_200, 0, x_199); +lean_ctor_set(x_200, 1, x_182); +return x_200; } else { -lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; uint8_t x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; -x_210 = l_Lean_Elab_instInhabitedInfoTree; -x_211 = l_Lean_PersistentArray_get_x21___rarg(x_210, x_194, x_196); -x_212 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_212, 0, x_211); -x_213 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__10; -x_214 = 0; -x_215 = lean_alloc_ctor(0, 3, 1); -lean_ctor_set(x_215, 0, x_213); -lean_ctor_set(x_215, 1, x_8); -lean_ctor_set(x_215, 2, x_212); -lean_ctor_set_uint8(x_215, sizeof(void*)*3, x_214); -x_216 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_216, 0, x_215); -lean_ctor_set(x_216, 1, x_201); -if (lean_is_scalar(x_192)) { - x_217 = lean_alloc_ctor(0, 2, 0); +lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; uint8_t x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; +x_201 = l_Lean_Elab_instInhabitedInfoTree; +x_202 = l_Lean_PersistentArray_get_x21___rarg(x_201, x_185, x_187); +x_203 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_203, 0, x_202); +x_204 = l_Lean_Language_Lean_process_processHeader___lambda__3___closed__10; +x_205 = 0; +x_206 = lean_alloc_ctor(0, 3, 1); +lean_ctor_set(x_206, 0, x_204); +lean_ctor_set(x_206, 1, x_8); +lean_ctor_set(x_206, 2, x_203); +lean_ctor_set_uint8(x_206, sizeof(void*)*3, x_205); +x_207 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_207, 0, x_206); +lean_ctor_set(x_207, 1, x_192); +if (lean_is_scalar(x_183)) { + x_208 = lean_alloc_ctor(0, 2, 0); } else { - x_217 = x_192; + x_208 = x_183; } -lean_ctor_set(x_217, 0, x_216); -lean_ctor_set(x_217, 1, x_191); -return x_217; +lean_ctor_set(x_208, 0, x_207); +lean_ctor_set(x_208, 1, x_182); +return x_208; } } } else { -uint8_t x_218; +uint8_t x_209; lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -8551,28 +8995,28 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); lean_dec(x_2); -x_218 = !lean_is_exclusive(x_13); -if (x_218 == 0) +x_209 = !lean_is_exclusive(x_13); +if (x_209 == 0) { return x_13; } else { -lean_object* x_219; lean_object* x_220; lean_object* x_221; -x_219 = lean_ctor_get(x_13, 0); -x_220 = lean_ctor_get(x_13, 1); -lean_inc(x_220); -lean_inc(x_219); +lean_object* x_210; lean_object* x_211; lean_object* x_212; +x_210 = lean_ctor_get(x_13, 0); +x_211 = lean_ctor_get(x_13, 1); +lean_inc(x_211); +lean_inc(x_210); lean_dec(x_13); -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; +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; } } } } -static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__5___closed__1() { +static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__4___closed__1() { _start: { lean_object* x_1; lean_object* x_2; @@ -8581,17 +9025,17 @@ x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__5___closed__2() { +static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__4___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Language_Lean_process_processHeader___lambda__5___closed__1; +x_1 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__1; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static size_t _init_l_Lean_Language_Lean_process_processHeader___lambda__5___closed__3() { +static size_t _init_l_Lean_Language_Lean_process_processHeader___lambda__4___closed__3() { _start: { lean_object* x_1; size_t x_2; @@ -8600,14 +9044,14 @@ x_2 = lean_usize_of_nat(x_1); return x_2; } } -static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__5___closed__4() { +static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__4___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; size_t x_4; lean_object* x_5; -x_1 = l_Lean_Language_Lean_process_processHeader___lambda__5___closed__2; -x_2 = l_Lean_Language_Lean_process_processHeader___lambda__5___closed__1; +x_1 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__2; +x_2 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__1; x_3 = lean_unsigned_to_nat(0u); -x_4 = l_Lean_Language_Lean_process_processHeader___lambda__5___closed__3; +x_4 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__3; x_5 = lean_alloc_ctor(0, 4, sizeof(size_t)*1); lean_ctor_set(x_5, 0, x_1); lean_ctor_set(x_5, 1, x_2); @@ -8617,7 +9061,7 @@ lean_ctor_set_usize(x_5, 4, x_4); return x_5; } } -static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__5___closed__5() { +static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__4___closed__5() { _start: { lean_object* x_1; @@ -8625,7 +9069,7 @@ x_1 = l_Lean_trace_profiler_output; return x_1; } } -static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__5___closed__6() { +static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__4___closed__6() { _start: { lean_object* x_1; @@ -8633,17 +9077,17 @@ x_1 = lean_mk_string_unchecked("Import", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__5___closed__7() { +static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__4___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Language_Lean_process_processHeader___lambda__5___closed__6; +x_2 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__5___closed__8() { +static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__4___closed__8() { _start: { lean_object* x_1; @@ -8651,26 +9095,26 @@ x_1 = lean_mk_string_unchecked("importing", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__5___closed__9() { +static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__4___closed__9() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Language_Lean_process_processHeader___lambda__5___closed__8; +x_1 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__8; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__5___closed__10() { +static lean_object* _init_l_Lean_Language_Lean_process_processHeader___lambda__4___closed__10() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Language_Lean_process_processHeader___lambda__5___closed__9; +x_1 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__9; x_2 = l_Lean_MessageData_ofFormat(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_processHeader___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, double x_10, double x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_processHeader___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, double x_10, double 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; @@ -8678,21 +9122,21 @@ x_15 = lean_ctor_get(x_1, 0); lean_inc(x_15); lean_dec(x_1); x_16 = lean_environment_set_main_module(x_2, x_15); -x_17 = l_Lean_Language_Lean_process_processHeader___lambda__5___closed__5; +x_17 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__5; x_18 = l_Lean_Option_get_x3f___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessages___spec__1(x_3, x_17); if (lean_obj_tag(x_18) == 0) { lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_19 = l_Lean_Language_Lean_process_processHeader___lambda__5___closed__4; +x_19 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__4; x_20 = lean_box(0); -x_21 = l_Lean_Language_Lean_process_processHeader___lambda__4(x_3, x_16, x_4, x_5, x_6, x_7, x_8, x_9, x_19, x_20, x_13, x_14); +x_21 = l_Lean_Language_Lean_process_processHeader___lambda__3(x_3, x_16, x_4, x_5, x_6, x_7, x_8, x_9, x_19, x_20, x_13, x_14); return x_21; } else { lean_object* x_22; uint8_t x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_dec(x_18); -x_22 = l_Lean_Language_Lean_process_processHeader___lambda__5___closed__7; +x_22 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__7; x_23 = 1; x_24 = l_Lean_Language_Lean_initFn____x40_Lean_Language_Lean___hyg_437____closed__4; x_25 = lean_alloc_ctor(0, 2, 17); @@ -8702,7 +9146,7 @@ lean_ctor_set_float(x_25, sizeof(void*)*2, x_10); lean_ctor_set_float(x_25, sizeof(void*)*2 + 8, x_11); lean_ctor_set_uint8(x_25, sizeof(void*)*2 + 16, x_23); x_26 = lean_box(0); -x_27 = l_Lean_Language_Lean_process_processHeader___lambda__5___closed__10; +x_27 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__10; x_28 = l_List_mapTR_loop___at_Lean_Language_Lean_process_processHeader___spec__1___closed__3; x_29 = lean_alloc_ctor(9, 3, 0); lean_ctor_set(x_29, 0, x_25); @@ -8719,12 +9163,12 @@ x_33 = lean_array_mk(x_32); x_34 = l_Array_toPArray_x27___rarg(x_33); lean_dec(x_33); x_35 = lean_box(0); -x_36 = l_Lean_Language_Lean_process_processHeader___lambda__4(x_3, x_16, x_4, x_5, x_6, x_7, x_8, x_9, x_34, x_35, x_13, x_14); +x_36 = l_Lean_Language_Lean_process_processHeader___lambda__3(x_3, x_16, x_4, x_5, x_6, x_7, x_8, x_9, x_34, x_35, x_13, x_14); return x_36; } } } -static double _init_l_Lean_Language_Lean_process_processHeader___lambda__6___closed__1() { +static double _init_l_Lean_Language_Lean_process_processHeader___lambda__5___closed__1() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; double x_4; @@ -8735,7 +9179,7 @@ x_4 = l_Float_ofScientific(x_1, x_2, x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_processHeader___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_processHeader___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; uint8_t x_11; lean_object* x_12; double x_13; double x_14; double x_15; lean_object* x_16; uint32_t x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; @@ -8749,7 +9193,7 @@ x_11 = 0; x_12 = lean_unsigned_to_nat(0u); x_13 = l_Float_ofScientific(x_9, x_11, x_12); lean_dec(x_9); -x_14 = l_Lean_Language_Lean_process_processHeader___lambda__6___closed__1; +x_14 = l_Lean_Language_Lean_process_processHeader___lambda__5___closed__1; x_15 = lean_float_div(x_13, x_14); x_16 = lean_ctor_get(x_5, 1); lean_inc(x_16); @@ -8797,7 +9241,7 @@ lean_object* x_36; lean_object* x_37; lean_free_object(x_31); lean_free_object(x_25); x_36 = lean_box(0); -x_37 = l_Lean_Language_Lean_process_processHeader___lambda__5(x_5, x_23, x_16, x_24, x_2, x_1, x_3, x_4, x_33, x_15, x_30, x_36, x_6, x_34); +x_37 = l_Lean_Language_Lean_process_processHeader___lambda__4(x_5, x_23, x_16, x_24, x_2, x_1, x_3, x_4, x_33, x_15, x_30, x_36, x_6, x_34); lean_dec(x_2); return x_37; } @@ -8813,7 +9257,7 @@ lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); x_38 = lean_box(0); -x_39 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__10; +x_39 = l_Lean_Language_Lean_process_processHeader___lambda__3___closed__10; x_40 = lean_alloc_ctor(0, 3, 1); lean_ctor_set(x_40, 0, x_39); lean_ctor_set(x_40, 1, x_33); @@ -8839,7 +9283,7 @@ if (x_43 == 0) lean_object* x_44; lean_object* x_45; lean_free_object(x_25); x_44 = lean_box(0); -x_45 = l_Lean_Language_Lean_process_processHeader___lambda__5(x_5, x_23, x_16, x_24, x_2, x_1, x_3, x_4, x_41, x_15, x_30, x_44, x_6, x_42); +x_45 = l_Lean_Language_Lean_process_processHeader___lambda__4(x_5, x_23, x_16, x_24, x_2, x_1, x_3, x_4, x_41, x_15, x_30, x_44, x_6, x_42); lean_dec(x_2); return x_45; } @@ -8855,7 +9299,7 @@ lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); x_46 = lean_box(0); -x_47 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__10; +x_47 = l_Lean_Language_Lean_process_processHeader___lambda__3___closed__10; x_48 = lean_alloc_ctor(0, 3, 1); lean_ctor_set(x_48, 0, x_47); lean_ctor_set(x_48, 1, x_41); @@ -8901,7 +9345,7 @@ if (x_58 == 0) lean_object* x_59; lean_object* x_60; lean_dec(x_57); x_59 = lean_box(0); -x_60 = l_Lean_Language_Lean_process_processHeader___lambda__5(x_5, x_23, x_16, x_24, x_2, x_1, x_3, x_4, x_55, x_15, x_53, x_59, x_6, x_56); +x_60 = l_Lean_Language_Lean_process_processHeader___lambda__4(x_5, x_23, x_16, x_24, x_2, x_1, x_3, x_4, x_55, x_15, x_53, x_59, x_6, x_56); lean_dec(x_2); return x_60; } @@ -8917,7 +9361,7 @@ lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); x_61 = lean_box(0); -x_62 = l_Lean_Language_Lean_process_processHeader___lambda__4___closed__10; +x_62 = l_Lean_Language_Lean_process_processHeader___lambda__3___closed__10; x_63 = lean_alloc_ctor(0, 3, 1); lean_ctor_set(x_63, 0, x_62); lean_ctor_set(x_63, 1, x_55); @@ -8967,7 +9411,7 @@ return x_69; } } } -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_processHeader___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_EXPORT lean_object* l_Lean_Language_Lean_process_processHeader___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { if (lean_obj_tag(x_5) == 0) @@ -8991,7 +9435,7 @@ lean_object* x_10; lean_object* x_11; x_10 = lean_ctor_get(x_5, 0); lean_inc(x_10); lean_dec(x_5); -x_11 = l_Lean_Language_Lean_process_processHeader___lambda__6(x_1, x_2, x_3, x_4, x_10, x_6, x_7); +x_11 = l_Lean_Language_Lean_process_processHeader___lambda__5(x_1, x_2, x_3, x_4, x_10, x_6, x_7); return x_11; } } @@ -9025,7 +9469,7 @@ x_12 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_processHeader___l lean_closure_set(x_12, 0, x_1); lean_closure_set(x_12, 1, x_2); lean_inc(x_4); -x_13 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_processHeader___lambda__7___boxed), 7, 4); +x_13 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_processHeader___lambda__6___boxed), 7, 4); lean_closure_set(x_13, 0, x_2); lean_closure_set(x_13, 1, x_6); lean_closure_set(x_13, 2, x_3); @@ -9042,18 +9486,18 @@ x_17 = l_Lean_Language_SnapshotTask_ofIO___rarg(x_11, x_16, x_5); return x_17; } } -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_processHeader___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_processHeader___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; -x_13 = l_Lean_Language_Lean_process_processHeader___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_13 = l_Lean_Language_Lean_process_processHeader___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_4); return x_13; } } -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_processHeader___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_processHeader___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: { double x_15; double x_16; lean_object* x_17; @@ -9061,27 +9505,27 @@ x_15 = lean_unbox_float(x_10); lean_dec(x_10); x_16 = lean_unbox_float(x_11); lean_dec(x_11); -x_17 = l_Lean_Language_Lean_process_processHeader___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_15, x_16, x_12, x_13, x_14); +x_17 = l_Lean_Language_Lean_process_processHeader___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_15, x_16, x_12, x_13, x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_5); return x_17; } } -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_processHeader___lambda__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_processHeader___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_Language_Lean_process_processHeader___lambda__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Lean_Language_Lean_process_processHeader___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_6); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_processHeader___lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Language_Lean_process_processHeader___lambda__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; -x_8 = l_Lean_Language_Lean_process_processHeader___lambda__7(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Lean_Language_Lean_process_processHeader___lambda__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_6); return x_8; } @@ -9311,7 +9755,7 @@ lean_object* x_7; x_7 = lean_io_promise_new(x_6); 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_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; lean_object* x_13; x_8 = lean_ctor_get(x_7, 0); lean_inc(x_8); x_9 = lean_ctor_get(x_7, 1); @@ -9322,190 +9766,182 @@ lean_ctor_set(x_10, 0, x_5); x_11 = lean_ctor_get(x_1, 0); lean_inc(x_11); lean_dec(x_1); +x_12 = 1; lean_inc(x_8); lean_inc(x_11); -x_12 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_processHeader___lambda__3), 6, 5); -lean_closure_set(x_12, 0, x_10); -lean_closure_set(x_12, 1, x_2); -lean_closure_set(x_12, 2, x_11); -lean_closure_set(x_12, 3, x_8); -lean_closure_set(x_12, 4, x_3); -x_13 = lean_alloc_closure((void*)(l_EIO_toBaseIO___rarg), 2, 1); -lean_closure_set(x_13, 0, x_12); -x_14 = l_Task_Priority_default; -x_15 = lean_io_as_task(x_13, x_14, x_9); -if (lean_obj_tag(x_15) == 0) +x_13 = l_Lean_Language_Lean_process_parseCmd(x_10, x_2, x_11, x_8, x_12, x_3, x_9); +if (lean_obj_tag(x_13) == 0) { -lean_object* x_16; uint8_t x_17; -x_16 = lean_ctor_get(x_4, 0); -lean_inc(x_16); +lean_object* x_14; uint8_t x_15; +x_14 = lean_ctor_get(x_4, 0); +lean_inc(x_14); lean_dec(x_4); -x_17 = !lean_is_exclusive(x_15); +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) { -lean_object* x_18; uint8_t x_19; -x_18 = lean_ctor_get(x_15, 0); +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; lean_object* x_27; lean_object* x_28; +x_18 = lean_ctor_get(x_14, 2); lean_dec(x_18); -x_19 = !lean_is_exclusive(x_16); -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; uint8_t x_28; lean_object* x_29; lean_object* x_30; -x_20 = lean_ctor_get(x_16, 2); -lean_dec(x_20); -x_21 = lean_ctor_get(x_16, 0); -lean_dec(x_21); -x_22 = lean_box(0); -x_23 = lean_io_promise_result(x_8); -x_24 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_24, 0, x_22); -lean_ctor_set(x_24, 1, x_23); -x_25 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_25, 0, x_11); -lean_ctor_set(x_25, 1, x_24); -x_26 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_26, 0, x_25); -x_27 = l_Lean_Language_Lean_process_parseHeader___lambda__3___closed__3; -x_28 = 0; -lean_ctor_set(x_16, 2, x_22); -lean_ctor_set(x_16, 0, x_27); -lean_ctor_set_uint8(x_16, sizeof(void*)*3, x_28); -x_29 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_29, 0, x_16); -lean_ctor_set(x_29, 1, x_26); -x_30 = l_Lean_Language_SnapshotTask_pure___rarg(x_29); -lean_ctor_set(x_15, 0, x_30); -return x_15; +x_19 = lean_ctor_get(x_14, 0); +lean_dec(x_19); +x_20 = lean_box(0); +x_21 = lean_io_promise_result(x_8); +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_11); +lean_ctor_set(x_23, 1, x_22); +x_24 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_24, 0, x_23); +x_25 = l_Lean_Language_Lean_process_parseHeader___lambda__3___closed__3; +x_26 = 0; +lean_ctor_set(x_14, 2, x_20); +lean_ctor_set(x_14, 0, x_25); +lean_ctor_set_uint8(x_14, sizeof(void*)*3, x_26); +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_14); +lean_ctor_set(x_27, 1, x_24); +x_28 = l_Lean_Language_SnapshotTask_pure___rarg(x_27); +lean_ctor_set(x_13, 0, x_28); +return x_13; } else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; uint8_t x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_31 = lean_ctor_get(x_16, 1); -lean_inc(x_31); -lean_dec(x_16); -x_32 = lean_box(0); -x_33 = lean_io_promise_result(x_8); -x_34 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_34, 0, x_32); -lean_ctor_set(x_34, 1, x_33); -x_35 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_35, 0, x_11); -lean_ctor_set(x_35, 1, x_34); -x_36 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_36, 0, x_35); -x_37 = l_Lean_Language_Lean_process_parseHeader___lambda__3___closed__3; -x_38 = 0; -x_39 = lean_alloc_ctor(0, 3, 1); -lean_ctor_set(x_39, 0, x_37); -lean_ctor_set(x_39, 1, x_31); -lean_ctor_set(x_39, 2, x_32); -lean_ctor_set_uint8(x_39, sizeof(void*)*3, 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_36); -x_41 = l_Lean_Language_SnapshotTask_pure___rarg(x_40); -lean_ctor_set(x_15, 0, x_41); -return x_15; +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_29 = lean_ctor_get(x_14, 1); +lean_inc(x_29); +lean_dec(x_14); +x_30 = lean_box(0); +x_31 = lean_io_promise_result(x_8); +x_32 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_31); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_11); +lean_ctor_set(x_33, 1, x_32); +x_34 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_34, 0, x_33); +x_35 = l_Lean_Language_Lean_process_parseHeader___lambda__3___closed__3; +x_36 = 0; +x_37 = lean_alloc_ctor(0, 3, 1); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_29); +lean_ctor_set(x_37, 2, x_30); +lean_ctor_set_uint8(x_37, sizeof(void*)*3, 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_34); +x_39 = l_Lean_Language_SnapshotTask_pure___rarg(x_38); +lean_ctor_set(x_13, 0, x_39); +return x_13; } } 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; uint8_t x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_42 = lean_ctor_get(x_15, 1); -lean_inc(x_42); -lean_dec(x_15); -x_43 = lean_ctor_get(x_16, 1); -lean_inc(x_43); -if (lean_is_exclusive(x_16)) { - lean_ctor_release(x_16, 0); - lean_ctor_release(x_16, 1); - lean_ctor_release(x_16, 2); - x_44 = x_16; +lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_40 = lean_ctor_get(x_13, 1); +lean_inc(x_40); +lean_dec(x_13); +x_41 = lean_ctor_get(x_14, 1); +lean_inc(x_41); +if (lean_is_exclusive(x_14)) { + lean_ctor_release(x_14, 0); + lean_ctor_release(x_14, 1); + lean_ctor_release(x_14, 2); + x_42 = x_14; } else { - lean_dec_ref(x_16); - x_44 = lean_box(0); + lean_dec_ref(x_14); + x_42 = lean_box(0); } -x_45 = lean_box(0); -x_46 = lean_io_promise_result(x_8); -x_47 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_47, 0, x_45); -lean_ctor_set(x_47, 1, x_46); -x_48 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_48, 0, x_11); -lean_ctor_set(x_48, 1, x_47); -x_49 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_49, 0, x_48); -x_50 = l_Lean_Language_Lean_process_parseHeader___lambda__3___closed__3; -x_51 = 0; -if (lean_is_scalar(x_44)) { - x_52 = lean_alloc_ctor(0, 3, 1); +x_43 = lean_box(0); +x_44 = lean_io_promise_result(x_8); +x_45 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_45, 0, x_43); +lean_ctor_set(x_45, 1, x_44); +x_46 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_46, 0, x_11); +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_Lean_Language_Lean_process_parseHeader___lambda__3___closed__3; +x_49 = 0; +if (lean_is_scalar(x_42)) { + x_50 = lean_alloc_ctor(0, 3, 1); } else { - x_52 = x_44; + x_50 = x_42; } -lean_ctor_set(x_52, 0, x_50); -lean_ctor_set(x_52, 1, x_43); -lean_ctor_set(x_52, 2, x_45); -lean_ctor_set_uint8(x_52, sizeof(void*)*3, x_51); +lean_ctor_set(x_50, 0, x_48); +lean_ctor_set(x_50, 1, x_41); +lean_ctor_set(x_50, 2, x_43); +lean_ctor_set_uint8(x_50, sizeof(void*)*3, 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_47); +x_52 = l_Lean_Language_SnapshotTask_pure___rarg(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_49); -x_54 = l_Lean_Language_SnapshotTask_pure___rarg(x_53); -x_55 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_55, 0, x_54); -lean_ctor_set(x_55, 1, x_42); -return x_55; +lean_ctor_set(x_53, 1, x_40); +return x_53; } } else { -uint8_t x_56; +uint8_t x_54; lean_dec(x_11); lean_dec(x_8); lean_dec(x_4); -x_56 = !lean_is_exclusive(x_15); -if (x_56 == 0) +x_54 = !lean_is_exclusive(x_13); +if (x_54 == 0) { -return x_15; +return x_13; } else { -lean_object* x_57; lean_object* x_58; lean_object* x_59; -x_57 = lean_ctor_get(x_15, 0); -x_58 = lean_ctor_get(x_15, 1); -lean_inc(x_58); -lean_inc(x_57); -lean_dec(x_15); -x_59 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_59, 0, x_57); -lean_ctor_set(x_59, 1, x_58); -return x_59; +lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_55 = lean_ctor_get(x_13, 0); +x_56 = lean_ctor_get(x_13, 1); +lean_inc(x_56); +lean_inc(x_55); +lean_dec(x_13); +x_57 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_57, 0, x_55); +lean_ctor_set(x_57, 1, x_56); +return x_57; } } } else { -uint8_t x_60; +uint8_t x_58; lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_60 = !lean_is_exclusive(x_7); -if (x_60 == 0) +x_58 = !lean_is_exclusive(x_7); +if (x_58 == 0) { return x_7; } else { -lean_object* x_61; lean_object* x_62; lean_object* x_63; -x_61 = lean_ctor_get(x_7, 0); -x_62 = lean_ctor_get(x_7, 1); -lean_inc(x_62); -lean_inc(x_61); +lean_object* x_59; lean_object* x_60; lean_object* x_61; +x_59 = lean_ctor_get(x_7, 0); +x_60 = lean_ctor_get(x_7, 1); +lean_inc(x_60); +lean_inc(x_59); lean_dec(x_7); -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; +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; } } } @@ -11487,234 +11923,243 @@ lean_dec(x_6); x_9 = lean_box(0); if (lean_obj_tag(x_4) == 0) { -lean_object* x_10; lean_object* x_11; +uint8_t x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_10 = 1; +x_11 = lean_box(x_10); lean_inc(x_7); -x_10 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_parseCmd), 6, 4); -lean_closure_set(x_10, 0, x_9); -lean_closure_set(x_10, 1, x_2); -lean_closure_set(x_10, 2, x_3); -lean_closure_set(x_10, 3, x_7); -x_11 = l_Lean_Language_Lean_LeanProcessingM_run___rarg(x_10, x_9, x_9, x_1, x_8); -if (lean_obj_tag(x_11) == 0) +x_12 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_parseCmd___boxed), 7, 5); +lean_closure_set(x_12, 0, x_9); +lean_closure_set(x_12, 1, x_2); +lean_closure_set(x_12, 2, x_3); +lean_closure_set(x_12, 3, x_7); +lean_closure_set(x_12, 4, x_11); +x_13 = l_Lean_Language_Lean_LeanProcessingM_run___rarg(x_12, x_9, x_9, x_1, x_8); +if (lean_obj_tag(x_13) == 0) { -uint8_t x_12; -x_12 = !lean_is_exclusive(x_11); -if (x_12 == 0) +uint8_t x_14; +x_14 = !lean_is_exclusive(x_13); +if (x_14 == 0) { -lean_object* x_13; lean_object* x_14; -x_13 = lean_ctor_get(x_11, 0); -lean_dec(x_13); -x_14 = lean_io_promise_result(x_7); -lean_ctor_set(x_11, 0, x_14); -return x_11; +lean_object* x_15; lean_object* x_16; +x_15 = lean_ctor_get(x_13, 0); +lean_dec(x_15); +x_16 = lean_io_promise_result(x_7); +lean_ctor_set(x_13, 0, x_16); +return x_13; } else { -lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = lean_ctor_get(x_11, 1); -lean_inc(x_15); -lean_dec(x_11); -x_16 = lean_io_promise_result(x_7); -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_16); -lean_ctor_set(x_17, 1, x_15); -return x_17; +lean_object* x_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_io_promise_result(x_7); +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set(x_19, 1, x_17); +return x_19; } } else { -uint8_t x_18; +uint8_t x_20; lean_dec(x_7); -x_18 = !lean_is_exclusive(x_11); -if (x_18 == 0) +x_20 = !lean_is_exclusive(x_13); +if (x_20 == 0) { -return x_11; +return x_13; } 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_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_13, 0); +x_22 = lean_ctor_get(x_13, 1); +lean_inc(x_22); +lean_inc(x_21); +lean_dec(x_13); +x_23 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_23, 0, x_21); +lean_ctor_set(x_23, 1, x_22); +return x_23; } } } else { -uint8_t x_22; -x_22 = !lean_is_exclusive(x_4); -if (x_22 == 0) +uint8_t x_24; +x_24 = !lean_is_exclusive(x_4); +if (x_24 == 0) { -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_23 = lean_ctor_get(x_4, 0); -x_24 = lean_ctor_get(x_23, 1); -lean_inc(x_24); -lean_ctor_set(x_4, 0, x_24); -lean_inc(x_7); -x_25 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_parseCmd), 6, 4); -lean_closure_set(x_25, 0, x_4); -lean_closure_set(x_25, 1, x_2); -lean_closure_set(x_25, 2, x_3); -lean_closure_set(x_25, 3, x_7); -x_26 = lean_ctor_get(x_23, 0); +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; +x_25 = lean_ctor_get(x_4, 0); +x_26 = lean_ctor_get(x_25, 1); lean_inc(x_26); -lean_dec(x_23); -x_27 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_27, 0, x_26); -x_28 = l_Lean_Language_Lean_LeanProcessingM_run___rarg(x_25, x_27, x_9, x_1, x_8); -if (lean_obj_tag(x_28) == 0) +lean_ctor_set(x_4, 0, x_26); +x_27 = 1; +x_28 = lean_box(x_27); +lean_inc(x_7); +x_29 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_parseCmd___boxed), 7, 5); +lean_closure_set(x_29, 0, x_4); +lean_closure_set(x_29, 1, x_2); +lean_closure_set(x_29, 2, x_3); +lean_closure_set(x_29, 3, x_7); +lean_closure_set(x_29, 4, x_28); +x_30 = lean_ctor_get(x_25, 0); +lean_inc(x_30); +lean_dec(x_25); +x_31 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_31, 0, x_30); +x_32 = l_Lean_Language_Lean_LeanProcessingM_run___rarg(x_29, x_31, x_9, x_1, x_8); +if (lean_obj_tag(x_32) == 0) { -uint8_t x_29; -x_29 = !lean_is_exclusive(x_28); -if (x_29 == 0) +uint8_t x_33; +x_33 = !lean_is_exclusive(x_32); +if (x_33 == 0) { -lean_object* x_30; lean_object* x_31; -x_30 = lean_ctor_get(x_28, 0); -lean_dec(x_30); -x_31 = lean_io_promise_result(x_7); -lean_ctor_set(x_28, 0, x_31); -return x_28; +lean_object* x_34; lean_object* x_35; +x_34 = lean_ctor_get(x_32, 0); +lean_dec(x_34); +x_35 = lean_io_promise_result(x_7); +lean_ctor_set(x_32, 0, x_35); +return x_32; } else { -lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_32 = lean_ctor_get(x_28, 1); -lean_inc(x_32); -lean_dec(x_28); -x_33 = lean_io_promise_result(x_7); -x_34 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_34, 0, x_33); -lean_ctor_set(x_34, 1, x_32); -return x_34; +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_32, 1); +lean_inc(x_36); +lean_dec(x_32); +x_37 = lean_io_promise_result(x_7); +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_35; +uint8_t x_39; lean_dec(x_7); -x_35 = !lean_is_exclusive(x_28); -if (x_35 == 0) +x_39 = !lean_is_exclusive(x_32); +if (x_39 == 0) { -return x_28; +return x_32; } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_28, 0); -x_37 = lean_ctor_get(x_28, 1); -lean_inc(x_37); -lean_inc(x_36); -lean_dec(x_28); -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_40; lean_object* x_41; lean_object* x_42; +x_40 = lean_ctor_get(x_32, 0); +x_41 = lean_ctor_get(x_32, 1); +lean_inc(x_41); +lean_inc(x_40); +lean_dec(x_32); +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_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_39 = lean_ctor_get(x_4, 0); -lean_inc(x_39); +lean_object* x_43; lean_object* x_44; lean_object* x_45; uint8_t x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_43 = lean_ctor_get(x_4, 0); +lean_inc(x_43); lean_dec(x_4); -x_40 = lean_ctor_get(x_39, 1); -lean_inc(x_40); -x_41 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_41, 0, x_40); +x_44 = lean_ctor_get(x_43, 1); +lean_inc(x_44); +x_45 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_45, 0, x_44); +x_46 = 1; +x_47 = lean_box(x_46); lean_inc(x_7); -x_42 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_parseCmd), 6, 4); -lean_closure_set(x_42, 0, x_41); -lean_closure_set(x_42, 1, x_2); -lean_closure_set(x_42, 2, x_3); -lean_closure_set(x_42, 3, x_7); -x_43 = lean_ctor_get(x_39, 0); -lean_inc(x_43); -lean_dec(x_39); -x_44 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_44, 0, x_43); -x_45 = l_Lean_Language_Lean_LeanProcessingM_run___rarg(x_42, x_44, x_9, x_1, x_8); -if (lean_obj_tag(x_45) == 0) +x_48 = lean_alloc_closure((void*)(l_Lean_Language_Lean_process_parseCmd___boxed), 7, 5); +lean_closure_set(x_48, 0, x_45); +lean_closure_set(x_48, 1, x_2); +lean_closure_set(x_48, 2, x_3); +lean_closure_set(x_48, 3, x_7); +lean_closure_set(x_48, 4, x_47); +x_49 = lean_ctor_get(x_43, 0); +lean_inc(x_49); +lean_dec(x_43); +x_50 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_50, 0, x_49); +x_51 = l_Lean_Language_Lean_LeanProcessingM_run___rarg(x_48, x_50, x_9, x_1, x_8); +if (lean_obj_tag(x_51) == 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); -if (lean_is_exclusive(x_45)) { - lean_ctor_release(x_45, 0); - lean_ctor_release(x_45, 1); - x_47 = x_45; +lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; +x_52 = lean_ctor_get(x_51, 1); +lean_inc(x_52); +if (lean_is_exclusive(x_51)) { + lean_ctor_release(x_51, 0); + lean_ctor_release(x_51, 1); + x_53 = x_51; } else { - lean_dec_ref(x_45); - x_47 = lean_box(0); + lean_dec_ref(x_51); + x_53 = lean_box(0); } -x_48 = lean_io_promise_result(x_7); -if (lean_is_scalar(x_47)) { - x_49 = lean_alloc_ctor(0, 2, 0); +x_54 = lean_io_promise_result(x_7); +if (lean_is_scalar(x_53)) { + x_55 = lean_alloc_ctor(0, 2, 0); } else { - x_49 = x_47; + x_55 = x_53; } -lean_ctor_set(x_49, 0, x_48); -lean_ctor_set(x_49, 1, x_46); -return x_49; +lean_ctor_set(x_55, 0, x_54); +lean_ctor_set(x_55, 1, x_52); +return x_55; } else { -lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; +lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_dec(x_7); -x_50 = lean_ctor_get(x_45, 0); -lean_inc(x_50); -x_51 = lean_ctor_get(x_45, 1); -lean_inc(x_51); -if (lean_is_exclusive(x_45)) { - lean_ctor_release(x_45, 0); - lean_ctor_release(x_45, 1); - x_52 = x_45; +x_56 = lean_ctor_get(x_51, 0); +lean_inc(x_56); +x_57 = lean_ctor_get(x_51, 1); +lean_inc(x_57); +if (lean_is_exclusive(x_51)) { + lean_ctor_release(x_51, 0); + lean_ctor_release(x_51, 1); + x_58 = x_51; } else { - lean_dec_ref(x_45); - x_52 = lean_box(0); + lean_dec_ref(x_51); + x_58 = lean_box(0); } -if (lean_is_scalar(x_52)) { - x_53 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_58)) { + x_59 = lean_alloc_ctor(1, 2, 0); } else { - x_53 = x_52; + x_59 = x_58; } -lean_ctor_set(x_53, 0, x_50); -lean_ctor_set(x_53, 1, x_51); -return x_53; +lean_ctor_set(x_59, 0, x_56); +lean_ctor_set(x_59, 1, x_57); +return x_59; } } } } else { -uint8_t x_54; +uint8_t x_60; lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_54 = !lean_is_exclusive(x_6); -if (x_54 == 0) +x_60 = !lean_is_exclusive(x_6); +if (x_60 == 0) { return x_6; } else { -lean_object* x_55; lean_object* x_56; lean_object* x_57; -x_55 = lean_ctor_get(x_6, 0); -x_56 = lean_ctor_get(x_6, 1); -lean_inc(x_56); -lean_inc(x_55); +lean_object* x_61; lean_object* x_62; lean_object* x_63; +x_61 = lean_ctor_get(x_6, 0); +x_62 = lean_ctor_get(x_6, 1); +lean_inc(x_62); +lean_inc(x_61); lean_dec(x_6); -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; +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; } } } @@ -11974,16 +12419,18 @@ l_Lean_Language_Lean_process_parseCmd___lambda__2___closed__4 = _init_l_Lean_Lan lean_mark_persistent(l_Lean_Language_Lean_process_parseCmd___lambda__2___closed__4); l_Lean_Language_Lean_process_parseCmd___lambda__3___closed__1 = _init_l_Lean_Language_Lean_process_parseCmd___lambda__3___closed__1(); lean_mark_persistent(l_Lean_Language_Lean_process_parseCmd___lambda__3___closed__1); +l_Lean_Language_Lean_process_parseCmd___lambda__4___closed__1 = _init_l_Lean_Language_Lean_process_parseCmd___lambda__4___closed__1(); +lean_mark_persistent(l_Lean_Language_Lean_process_parseCmd___lambda__4___closed__1); l_Lean_Language_Lean_process_parseCmd___lambda__5___closed__1 = _init_l_Lean_Language_Lean_process_parseCmd___lambda__5___closed__1(); lean_mark_persistent(l_Lean_Language_Lean_process_parseCmd___lambda__5___closed__1); +l_Lean_Language_Lean_process_parseCmd___lambda__5___closed__2 = _init_l_Lean_Language_Lean_process_parseCmd___lambda__5___closed__2(); +lean_mark_persistent(l_Lean_Language_Lean_process_parseCmd___lambda__5___closed__2); +l_Lean_Language_Lean_process_parseCmd___lambda__5___closed__3 = _init_l_Lean_Language_Lean_process_parseCmd___lambda__5___closed__3(); +lean_mark_persistent(l_Lean_Language_Lean_process_parseCmd___lambda__5___closed__3); l_Lean_Language_Lean_process_parseCmd___lambda__7___closed__1 = _init_l_Lean_Language_Lean_process_parseCmd___lambda__7___closed__1(); lean_mark_persistent(l_Lean_Language_Lean_process_parseCmd___lambda__7___closed__1); -l_Lean_Language_Lean_process_parseCmd___closed__1 = _init_l_Lean_Language_Lean_process_parseCmd___closed__1(); -lean_mark_persistent(l_Lean_Language_Lean_process_parseCmd___closed__1); -l_Lean_Language_Lean_process_parseCmd___closed__2 = _init_l_Lean_Language_Lean_process_parseCmd___closed__2(); -lean_mark_persistent(l_Lean_Language_Lean_process_parseCmd___closed__2); -l_Lean_Language_Lean_process_parseCmd___closed__3 = _init_l_Lean_Language_Lean_process_parseCmd___closed__3(); -lean_mark_persistent(l_Lean_Language_Lean_process_parseCmd___closed__3); +l_Lean_Language_Lean_process_parseCmd___lambda__9___closed__1 = _init_l_Lean_Language_Lean_process_parseCmd___lambda__9___closed__1(); +lean_mark_persistent(l_Lean_Language_Lean_process_parseCmd___lambda__9___closed__1); l_List_mapTR_loop___at_Lean_Language_Lean_process_processHeader___spec__1___closed__1 = _init_l_List_mapTR_loop___at_Lean_Language_Lean_process_processHeader___spec__1___closed__1(); lean_mark_persistent(l_List_mapTR_loop___at_Lean_Language_Lean_process_processHeader___spec__1___closed__1); l_List_mapTR_loop___at_Lean_Language_Lean_process_processHeader___spec__1___closed__2 = _init_l_List_mapTR_loop___at_Lean_Language_Lean_process_processHeader___spec__1___closed__2(); @@ -11992,12 +12439,31 @@ l_List_mapTR_loop___at_Lean_Language_Lean_process_processHeader___spec__1___clos lean_mark_persistent(l_List_mapTR_loop___at_Lean_Language_Lean_process_processHeader___spec__1___closed__3); l_List_mapTR_loop___at_Lean_Language_Lean_process_processHeader___spec__1___closed__4 = _init_l_List_mapTR_loop___at_Lean_Language_Lean_process_processHeader___spec__1___closed__4(); lean_mark_persistent(l_List_mapTR_loop___at_Lean_Language_Lean_process_processHeader___spec__1___closed__4); +l_Lean_Language_Lean_process_processHeader___lambda__3___closed__1 = _init_l_Lean_Language_Lean_process_processHeader___lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Language_Lean_process_processHeader___lambda__3___closed__1); +l_Lean_Language_Lean_process_processHeader___lambda__3___closed__2 = _init_l_Lean_Language_Lean_process_processHeader___lambda__3___closed__2(); +lean_mark_persistent(l_Lean_Language_Lean_process_processHeader___lambda__3___closed__2); +l_Lean_Language_Lean_process_processHeader___lambda__3___closed__3 = _init_l_Lean_Language_Lean_process_processHeader___lambda__3___closed__3(); +lean_mark_persistent(l_Lean_Language_Lean_process_processHeader___lambda__3___closed__3); +l_Lean_Language_Lean_process_processHeader___lambda__3___closed__4 = _init_l_Lean_Language_Lean_process_processHeader___lambda__3___closed__4(); +lean_mark_persistent(l_Lean_Language_Lean_process_processHeader___lambda__3___closed__4); +l_Lean_Language_Lean_process_processHeader___lambda__3___closed__5 = _init_l_Lean_Language_Lean_process_processHeader___lambda__3___closed__5(); +lean_mark_persistent(l_Lean_Language_Lean_process_processHeader___lambda__3___closed__5); +l_Lean_Language_Lean_process_processHeader___lambda__3___closed__6 = _init_l_Lean_Language_Lean_process_processHeader___lambda__3___closed__6(); +lean_mark_persistent(l_Lean_Language_Lean_process_processHeader___lambda__3___closed__6); +l_Lean_Language_Lean_process_processHeader___lambda__3___closed__7 = _init_l_Lean_Language_Lean_process_processHeader___lambda__3___closed__7(); +lean_mark_persistent(l_Lean_Language_Lean_process_processHeader___lambda__3___closed__7); +l_Lean_Language_Lean_process_processHeader___lambda__3___closed__8 = _init_l_Lean_Language_Lean_process_processHeader___lambda__3___closed__8(); +lean_mark_persistent(l_Lean_Language_Lean_process_processHeader___lambda__3___closed__8); +l_Lean_Language_Lean_process_processHeader___lambda__3___closed__9 = _init_l_Lean_Language_Lean_process_processHeader___lambda__3___closed__9(); +lean_mark_persistent(l_Lean_Language_Lean_process_processHeader___lambda__3___closed__9); +l_Lean_Language_Lean_process_processHeader___lambda__3___closed__10 = _init_l_Lean_Language_Lean_process_processHeader___lambda__3___closed__10(); +lean_mark_persistent(l_Lean_Language_Lean_process_processHeader___lambda__3___closed__10); l_Lean_Language_Lean_process_processHeader___lambda__4___closed__1 = _init_l_Lean_Language_Lean_process_processHeader___lambda__4___closed__1(); lean_mark_persistent(l_Lean_Language_Lean_process_processHeader___lambda__4___closed__1); l_Lean_Language_Lean_process_processHeader___lambda__4___closed__2 = _init_l_Lean_Language_Lean_process_processHeader___lambda__4___closed__2(); lean_mark_persistent(l_Lean_Language_Lean_process_processHeader___lambda__4___closed__2); l_Lean_Language_Lean_process_processHeader___lambda__4___closed__3 = _init_l_Lean_Language_Lean_process_processHeader___lambda__4___closed__3(); -lean_mark_persistent(l_Lean_Language_Lean_process_processHeader___lambda__4___closed__3); l_Lean_Language_Lean_process_processHeader___lambda__4___closed__4 = _init_l_Lean_Language_Lean_process_processHeader___lambda__4___closed__4(); lean_mark_persistent(l_Lean_Language_Lean_process_processHeader___lambda__4___closed__4); l_Lean_Language_Lean_process_processHeader___lambda__4___closed__5 = _init_l_Lean_Language_Lean_process_processHeader___lambda__4___closed__5(); @@ -12013,25 +12479,6 @@ lean_mark_persistent(l_Lean_Language_Lean_process_processHeader___lambda__4___cl l_Lean_Language_Lean_process_processHeader___lambda__4___closed__10 = _init_l_Lean_Language_Lean_process_processHeader___lambda__4___closed__10(); lean_mark_persistent(l_Lean_Language_Lean_process_processHeader___lambda__4___closed__10); l_Lean_Language_Lean_process_processHeader___lambda__5___closed__1 = _init_l_Lean_Language_Lean_process_processHeader___lambda__5___closed__1(); -lean_mark_persistent(l_Lean_Language_Lean_process_processHeader___lambda__5___closed__1); -l_Lean_Language_Lean_process_processHeader___lambda__5___closed__2 = _init_l_Lean_Language_Lean_process_processHeader___lambda__5___closed__2(); -lean_mark_persistent(l_Lean_Language_Lean_process_processHeader___lambda__5___closed__2); -l_Lean_Language_Lean_process_processHeader___lambda__5___closed__3 = _init_l_Lean_Language_Lean_process_processHeader___lambda__5___closed__3(); -l_Lean_Language_Lean_process_processHeader___lambda__5___closed__4 = _init_l_Lean_Language_Lean_process_processHeader___lambda__5___closed__4(); -lean_mark_persistent(l_Lean_Language_Lean_process_processHeader___lambda__5___closed__4); -l_Lean_Language_Lean_process_processHeader___lambda__5___closed__5 = _init_l_Lean_Language_Lean_process_processHeader___lambda__5___closed__5(); -lean_mark_persistent(l_Lean_Language_Lean_process_processHeader___lambda__5___closed__5); -l_Lean_Language_Lean_process_processHeader___lambda__5___closed__6 = _init_l_Lean_Language_Lean_process_processHeader___lambda__5___closed__6(); -lean_mark_persistent(l_Lean_Language_Lean_process_processHeader___lambda__5___closed__6); -l_Lean_Language_Lean_process_processHeader___lambda__5___closed__7 = _init_l_Lean_Language_Lean_process_processHeader___lambda__5___closed__7(); -lean_mark_persistent(l_Lean_Language_Lean_process_processHeader___lambda__5___closed__7); -l_Lean_Language_Lean_process_processHeader___lambda__5___closed__8 = _init_l_Lean_Language_Lean_process_processHeader___lambda__5___closed__8(); -lean_mark_persistent(l_Lean_Language_Lean_process_processHeader___lambda__5___closed__8); -l_Lean_Language_Lean_process_processHeader___lambda__5___closed__9 = _init_l_Lean_Language_Lean_process_processHeader___lambda__5___closed__9(); -lean_mark_persistent(l_Lean_Language_Lean_process_processHeader___lambda__5___closed__9); -l_Lean_Language_Lean_process_processHeader___lambda__5___closed__10 = _init_l_Lean_Language_Lean_process_processHeader___lambda__5___closed__10(); -lean_mark_persistent(l_Lean_Language_Lean_process_processHeader___lambda__5___closed__10); -l_Lean_Language_Lean_process_processHeader___lambda__6___closed__1 = _init_l_Lean_Language_Lean_process_processHeader___lambda__6___closed__1(); l_Lean_Language_Lean_process_processHeader___closed__1 = _init_l_Lean_Language_Lean_process_processHeader___closed__1(); lean_mark_persistent(l_Lean_Language_Lean_process_processHeader___closed__1); l_Lean_Language_Lean_process_parseHeader___lambda__3___closed__1 = _init_l_Lean_Language_Lean_process_parseHeader___lambda__3___closed__1(); diff --git a/stage0/stdlib/Lean/Language/Lean/Types.c b/stage0/stdlib/Lean/Language/Lean/Types.c index d6c494f83544..242bce031457 100644 --- a/stage0/stdlib/Lean/Language/Lean/Types.c +++ b/stage0/stdlib/Lean/Language/Lean/Types.c @@ -27,6 +27,7 @@ LEAN_EXPORT lean_object* l_Lean_Language_Lean_HeaderParsedSnapshot_processedResu static lean_object* l_Lean_Language_Lean_instToSnapshotTreeCommandParsedSnapshot_go___closed__3; static lean_object* l_Lean_Language_Lean_instToSnapshotTreeCommandParsedSnapshot_go___closed__2; LEAN_EXPORT lean_object* l_Lean_Language_Lean_CommandParsedSnapshot_nextCmdSnap_x3f___boxed(lean_object*); +lean_object* lean_thunk_get_own(lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_Lean_HeaderParsedSnapshot_processedResult___lambda__1___boxed(lean_object*); static lean_object* l_Lean_Language_Lean_instToSnapshotTreeCommandParsedSnapshot_go___closed__1; LEAN_EXPORT lean_object* l_Lean_Language_Lean_instToSnapshotTreeCommandParsedSnapshot_go___lambda__2(lean_object*); @@ -144,10 +145,10 @@ return x_2; LEAN_EXPORT lean_object* l_Lean_Language_Lean_instToSnapshotTreeCommandParsedSnapshot_go___lambda__1(lean_object* x_1) { _start: { -lean_object* x_2; +lean_object* x_2; lean_object* x_3; x_2 = lean_ctor_get(x_1, 1); -lean_inc(x_2); -return x_2; +x_3 = lean_thunk_get_own(x_2); +return x_3; } } LEAN_EXPORT lean_object* l_Lean_Language_Lean_instToSnapshotTreeCommandParsedSnapshot_go___lambda__2(lean_object* x_1) { diff --git a/stage0/stdlib/Lean/LazyInitExtension.c b/stage0/stdlib/Lean/LazyInitExtension.c deleted file mode 100644 index fd852129ca29..000000000000 --- a/stage0/stdlib/Lean/LazyInitExtension.c +++ /dev/null @@ -1,322 +0,0 @@ -// Lean compiler output -// Module: Lean.LazyInitExtension -// Imports: Lean.MonadEnv -#include -#if defined(__clang__) -#pragma clang diagnostic ignored "-Wunused-parameter" -#pragma clang diagnostic ignored "-Wunused-label" -#elif defined(__GNUC__) && !defined(__CLANG__) -#pragma GCC diagnostic ignored "-Wunused-parameter" -#pragma GCC diagnostic ignored "-Wunused-label" -#pragma GCC diagnostic ignored "-Wunused-but-set-variable" -#endif -#ifdef __cplusplus -extern "C" { -#endif -LEAN_EXPORT lean_object* l_Lean_instInhabitedLazyInitExtensionOfMonad(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___rarg___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_EnvExtensionInterfaceUnsafe_registerExt___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_registerLazyInitExtension___rarg(lean_object*, lean_object*); -lean_object* l_Lean_EnvExtensionInterfaceUnsafe_instInhabitedExt___lambda__1(lean_object*); -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___rarg___lambda__1(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_EnvExtension_getState___rarg(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_registerLazyInitExtension___rarg___closed__1; -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_EStateM_pure___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_registerLazyInitExtension(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_instInhabitedLazyInitExtensionOfMonad___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___rarg___lambda__2(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_instInhabitedLazyInitExtensionOfMonad___rarg___closed__2; -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get(lean_object*, lean_object*); -lean_object* l_Lean_EnvExtension_setState___rarg(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_instInhabitedLazyInitExtensionOfMonad___rarg___closed__1; -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* _init_l_Lean_instInhabitedLazyInitExtensionOfMonad___rarg___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_EnvExtensionInterfaceUnsafe_instInhabitedExt___lambda__1), 1, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_instInhabitedLazyInitExtensionOfMonad___rarg___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(0u); -x_2 = l_Lean_instInhabitedLazyInitExtensionOfMonad___rarg___closed__1; -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_instInhabitedLazyInitExtensionOfMonad___rarg(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_3 = lean_ctor_get(x_1, 0); -lean_inc(x_3); -lean_dec(x_1); -x_4 = lean_ctor_get(x_3, 1); -lean_inc(x_4); -lean_dec(x_3); -x_5 = lean_apply_2(x_4, lean_box(0), x_2); -x_6 = l_Lean_instInhabitedLazyInitExtensionOfMonad___rarg___closed__2; -x_7 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_7, 0, x_6); -lean_ctor_set(x_7, 1, x_5); -return x_7; -} -} -LEAN_EXPORT lean_object* l_Lean_instInhabitedLazyInitExtensionOfMonad(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Lean_instInhabitedLazyInitExtensionOfMonad___rarg), 2, 0); -return x_3; -} -} -static lean_object* _init_l_Lean_registerLazyInitExtension___rarg___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = lean_box(0); -x_2 = lean_alloc_closure((void*)(l_EStateM_pure___rarg), 2, 1); -lean_closure_set(x_2, 0, x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_registerLazyInitExtension___rarg(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; lean_object* x_4; -x_3 = l_Lean_registerLazyInitExtension___rarg___closed__1; -x_4 = l_Lean_EnvExtensionInterfaceUnsafe_registerExt___rarg(x_3, x_2); -if (lean_obj_tag(x_4) == 0) -{ -uint8_t x_5; -x_5 = !lean_is_exclusive(x_4); -if (x_5 == 0) -{ -lean_object* x_6; lean_object* x_7; -x_6 = lean_ctor_get(x_4, 0); -x_7 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_7, 0, x_6); -lean_ctor_set(x_7, 1, x_1); -lean_ctor_set(x_4, 0, x_7); -return x_4; -} -else -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_8 = lean_ctor_get(x_4, 0); -x_9 = lean_ctor_get(x_4, 1); -lean_inc(x_9); -lean_inc(x_8); -lean_dec(x_4); -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_8); -lean_ctor_set(x_10, 1, x_1); -x_11 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_11, 0, x_10); -lean_ctor_set(x_11, 1, x_9); -return x_11; -} -} -else -{ -uint8_t x_12; -lean_dec(x_1); -x_12 = !lean_is_exclusive(x_4); -if (x_12 == 0) -{ -return x_4; -} -else -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_ctor_get(x_4, 0); -x_14 = lean_ctor_get(x_4, 1); -lean_inc(x_14); -lean_inc(x_13); -lean_dec(x_4); -x_15 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_15, 0, x_13); -lean_ctor_set(x_15, 1, x_14); -return x_15; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_registerLazyInitExtension(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Lean_registerLazyInitExtension___rarg), 2, 0); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; lean_object* x_5; -x_4 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_4, 0, x_1); -x_5 = l_Lean_EnvExtension_setState___rarg(x_2, x_3, x_4); -return x_5; -} -} -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_4 = lean_ctor_get(x_1, 0); -lean_inc(x_4); -lean_dec(x_1); -x_5 = lean_ctor_get(x_4, 1); -lean_inc(x_5); -lean_dec(x_4); -x_6 = lean_apply_2(x_5, lean_box(0), x_2); -return x_6; -} -} -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; -x_6 = lean_ctor_get(x_1, 1); -lean_inc(x_6); -lean_dec(x_1); -lean_inc(x_5); -x_7 = lean_alloc_closure((void*)(l_Lean_LazyInitExtension_get___rarg___lambda__1___boxed), 3, 2); -lean_closure_set(x_7, 0, x_5); -lean_closure_set(x_7, 1, x_2); -x_8 = lean_apply_1(x_6, x_7); -x_9 = lean_alloc_closure((void*)(l_Lean_LazyInitExtension_get___rarg___lambda__2___boxed), 3, 2); -lean_closure_set(x_9, 0, x_3); -lean_closure_set(x_9, 1, x_5); -x_10 = lean_apply_4(x_4, lean_box(0), lean_box(0), x_8, x_9); -return x_10; -} -} -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_6 = lean_box(0); -x_7 = lean_ctor_get(x_1, 0); -lean_inc(x_7); -x_8 = l_Lean_EnvExtension_getState___rarg(x_6, x_7, x_5); -if (lean_obj_tag(x_8) == 0) -{ -lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_9 = lean_ctor_get(x_1, 1); -lean_inc(x_9); -lean_dec(x_1); -lean_inc(x_4); -x_10 = lean_alloc_closure((void*)(l_Lean_LazyInitExtension_get___rarg___lambda__3), 5, 4); -lean_closure_set(x_10, 0, x_2); -lean_closure_set(x_10, 1, x_7); -lean_closure_set(x_10, 2, x_3); -lean_closure_set(x_10, 3, x_4); -x_11 = lean_apply_4(x_4, lean_box(0), lean_box(0), x_9, x_10); -return x_11; -} -else -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -lean_dec(x_7); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -x_12 = lean_ctor_get(x_8, 0); -lean_inc(x_12); -lean_dec(x_8); -x_13 = lean_ctor_get(x_3, 0); -lean_inc(x_13); -lean_dec(x_3); -x_14 = lean_ctor_get(x_13, 1); -lean_inc(x_14); -lean_dec(x_13); -x_15 = lean_apply_2(x_14, lean_box(0), x_12); -return x_15; -} -} -} -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_4 = lean_ctor_get(x_2, 1); -lean_inc(x_4); -x_5 = lean_ctor_get(x_1, 0); -lean_inc(x_5); -lean_inc(x_4); -x_6 = lean_alloc_closure((void*)(l_Lean_LazyInitExtension_get___rarg___lambda__4___boxed), 5, 4); -lean_closure_set(x_6, 0, x_3); -lean_closure_set(x_6, 1, x_1); -lean_closure_set(x_6, 2, x_2); -lean_closure_set(x_6, 3, x_4); -x_7 = lean_apply_4(x_4, lean_box(0), lean_box(0), x_5, x_6); -return x_7; -} -} -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Lean_LazyInitExtension_get___rarg), 3, 0); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l_Lean_LazyInitExtension_get___rarg___lambda__1(x_1, x_2, x_3); -lean_dec(x_2); -return x_4; -} -} -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___rarg___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l_Lean_LazyInitExtension_get___rarg___lambda__2(x_1, x_2, x_3); -lean_dec(x_3); -return x_4; -} -} -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___rarg___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; -x_6 = l_Lean_LazyInitExtension_get___rarg___lambda__4(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_5); -return x_6; -} -} -lean_object* initialize_Lean_MonadEnv(uint8_t builtin, lean_object*); -static bool _G_initialized = false; -LEAN_EXPORT lean_object* initialize_Lean_LazyInitExtension(uint8_t builtin, lean_object* w) { -lean_object * res; -if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); -_G_initialized = true; -res = initialize_Lean_MonadEnv(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -l_Lean_instInhabitedLazyInitExtensionOfMonad___rarg___closed__1 = _init_l_Lean_instInhabitedLazyInitExtensionOfMonad___rarg___closed__1(); -lean_mark_persistent(l_Lean_instInhabitedLazyInitExtensionOfMonad___rarg___closed__1); -l_Lean_instInhabitedLazyInitExtensionOfMonad___rarg___closed__2 = _init_l_Lean_instInhabitedLazyInitExtensionOfMonad___rarg___closed__2(); -lean_mark_persistent(l_Lean_instInhabitedLazyInitExtensionOfMonad___rarg___closed__2); -l_Lean_registerLazyInitExtension___rarg___closed__1 = _init_l_Lean_registerLazyInitExtension___rarg___closed__1(); -lean_mark_persistent(l_Lean_registerLazyInitExtension___rarg___closed__1); -return lean_io_result_mk_ok(lean_box(0)); -} -#ifdef __cplusplus -} -#endif diff --git a/stage0/stdlib/Lean/Linter/ConstructorAsVariable.c b/stage0/stdlib/Lean/Linter/ConstructorAsVariable.c index ac66853ba0a9..19048351e0c2 100644 --- a/stage0/stdlib/Lean/Linter/ConstructorAsVariable.c +++ b/stage0/stdlib/Lean/Linter/ConstructorAsVariable.c @@ -13,126 +13,123 @@ #ifdef __cplusplus extern "C" { #endif -static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__2; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__4; static lean_object* l_Lean_Linter_constructorNameAsVariable___closed__1; -LEAN_EXPORT lean_object* l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__10(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__1; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_ConstructorAsVariable___hyg_8____closed__1; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__4(lean_object*, lean_object*); lean_object* l_Lean_PersistentArray_toArray___rarg(lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__5; lean_object* lean_whnf(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getHeadInfo(lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___boxed(lean_object*, lean_object*); uint64_t l___private_Lean_Syntax_0__String_hashRange____x40_Lean_Syntax___hyg_169_(lean_object*); -static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__4; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_uint64_to_usize(uint64_t); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___closed__1; LEAN_EXPORT lean_object* l_Lean_Linter_constructorNameAsVariable___elambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__1; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getId(lean_object*); uint8_t l___private_Lean_Syntax_0__String_beqRange____x40_Lean_Syntax___hyg_95_(lean_object*, lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__7___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_qpartition___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_mk_array(lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); -static lean_object* l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__1; -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__17(lean_object*, size_t, size_t, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___closed__1; lean_object* lean_array_fget(lean_object*, lean_object*); lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_constructorNameAsVariable___closed__3; LEAN_EXPORT lean_object* l_Lean_Linter_linter_constructorNameAsVariable; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__5(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_environment_find(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__17___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_logAt___at_Lean_Elab_Command_runLinters___spec__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__1; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_ConstructorAsVariable___hyg_8____closed__8; +LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Nat_nextPowerOfTwo_go(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_stringToMessageData(lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__8; lean_object* l_Lean_PersistentArray_toList___rarg(lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__6___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_string_dec_eq(lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__4; -static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__7; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__4; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__1___boxed(lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); lean_object* lean_local_ctx_find(lean_object*, lean_object*); lean_object* lean_st_ref_take(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__2; +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___lambda__1___boxed(lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__6___lambda__1___closed__1; uint64_t lean_uint64_shift_right(uint64_t, uint64_t); -LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_ConstructorAsVariable___hyg_8____closed__9; lean_object* lean_nat_div(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__2; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_ConstructorAsVariable___hyg_8____closed__2; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__11; lean_object* l_Lean_Elab_Info_updateContext_x3f(lean_object*, lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_ConstructorAsVariable___hyg_8____closed__6; +static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__5; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__2; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_PartialContextInfo_mergeIntoOuter_x3f(lean_object*, lean_object*); static lean_object* l_Lean_Linter_constructorNameAsVariable___elambda__1___closed__5; -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofFormat(lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__3; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__10; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__6; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__8; LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__7___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__7; lean_object* lean_st_mk_ref(lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__4___closed__1; -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__12; -static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__4; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__7; +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_inferType___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Elab_Command_instMonadCommandElabM; LEAN_EXPORT lean_object* l_Lean_Linter_constructorNameAsVariable___elambda__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_ConstructorAsVariable___hyg_8____closed__4; uint8_t l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__3; -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___lambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__12; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__10; lean_object* l_Lean_Elab_Command_addLinter(lean_object*, lean_object*); lean_object* l_Lean_Option_register___at_Lean_Elab_initFn____x40_Lean_Elab_AutoBound___hyg_6____spec__1(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__2; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_ConstructorAsVariable___hyg_8____closed__3; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__2(lean_object*); lean_object* l_Lean_LocalDecl_userName(lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__1; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__3; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__1; +LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Name_hasMacroScopes(lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_ConstructorAsVariable___hyg_8____closed__5; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_String_Range_contains(lean_object*, lean_object*, uint8_t); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12(lean_object*, lean_object*); lean_object* l_Lean_instantiateMVars___at___private_Lean_Meta_Basic_0__Lean_Meta_isClassApp_x3f___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__9; -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__6; +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__2; lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__3; static lean_object* l_Lean_Linter_constructorNameAsVariable___closed__2; -static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__6; -static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_getAppFn_x27(lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__3(lean_object*, lean_object*, lean_object*); uint64_t lean_uint64_xor(uint64_t, uint64_t); lean_object* lean_panic_fn(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__1; lean_object* lean_nat_sub(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_mul(lean_object*, lean_object*); lean_object* l_Lean_Syntax_getRange_x3f(lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_ConstructorAsVariable___hyg_8_(lean_object*); @@ -140,42 +137,44 @@ lean_object* l_Lean_Elab_TermInfo_runMetaM___rarg(lean_object*, lean_object*, le static lean_object* l_Lean_Linter_constructorNameAsVariable___elambda__1___closed__1; lean_object* l_Lean_Elab_Info_range_x3f(lean_object*); lean_object* l_List_reverse___rarg(lean_object*); +static lean_object* l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__1; size_t lean_usize_sub(size_t, size_t); lean_object* lean_array_mk(lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__11; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__7; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__5___closed__1; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_ConstructorAsVariable___hyg_8____closed__7; lean_object* lean_array_uget(lean_object*, size_t); size_t lean_array_size(lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__9; lean_object* lean_io_error_to_string(lean_object*); lean_object* l_instInhabitedOfMonad___rarg(lean_object*, lean_object*); lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); -static lean_object* l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__10___closed__1; -LEAN_EXPORT uint8_t l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___lambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___boxed(lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); static lean_object* l_Lean_Linter_constructorNameAsVariable___elambda__1___closed__2; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_constructorNameAsVariable___elambda__1___closed__4; uint8_t lean_nat_dec_le(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14(lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__4; lean_object* lean_nat_add(lean_object*, lean_object*); +static lean_object* l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__1; lean_object* l_Lean_Elab_Info_stx(lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_constructorNameAsVariable___elambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_ConstructorAsVariable___hyg_1340_(lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__3; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); lean_object* l_Lean_MessageData_ofName(lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__5; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__6; size_t lean_usize_land(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Linter_constructorNameAsVariable; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__6___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__5; -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___lambda__1___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Linter_constructorNameAsVariable___elambda__1___closed__3; static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_ConstructorAsVariable___hyg_8____closed__1() { _start: @@ -1199,7 +1198,7 @@ goto _start; } } } -static lean_object* _init_l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__10___closed__1() { +static lean_object* _init_l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -1209,17 +1208,17 @@ x_3 = l_instInhabitedOfMonad___rarg(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_5 = l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__10___closed__1; +x_5 = l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__1; x_6 = lean_panic_fn(x_5, x_1); x_7 = lean_apply_3(x_6, x_2, x_3, x_4); return x_7; } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { if (lean_obj_tag(x_4) == 0) @@ -1250,7 +1249,7 @@ lean_inc(x_6); lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_14 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9(x_1, x_2, x_3, x_12, x_6, x_7, x_8); +x_14 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8(x_1, x_2, x_3, x_12, x_6, x_7, x_8); if (lean_obj_tag(x_14) == 0) { lean_object* x_15; lean_object* x_16; @@ -1315,7 +1314,7 @@ lean_inc(x_6); lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_24 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9(x_1, x_2, x_3, x_22, x_6, x_7, x_8); +x_24 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8(x_1, x_2, x_3, x_22, x_6, x_7, x_8); if (lean_obj_tag(x_24) == 0) { lean_object* x_25; lean_object* x_26; lean_object* x_27; @@ -1367,7 +1366,7 @@ return x_32; } } } -static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__1() { +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__1() { _start: { lean_object* x_1; @@ -1375,7 +1374,7 @@ x_1 = lean_mk_string_unchecked("Lean.Server.InfoUtils", 21, 21); return x_1; } } -static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__2() { +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__2() { _start: { lean_object* x_1; @@ -1383,7 +1382,7 @@ x_1 = lean_mk_string_unchecked("Lean.Elab.InfoTree.visitM.go", 28, 28); return x_1; } } -static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__3() { +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__3() { _start: { lean_object* x_1; @@ -1391,20 +1390,20 @@ x_1 = lean_mk_string_unchecked("unexpected context-free info tree node", 38, 38) return x_1; } } -static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__4() { +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__1; -x_2 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__2; -x_3 = lean_unsigned_to_nat(56u); +x_1 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__1; +x_2 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__2; +x_3 = lean_unsigned_to_nat(62u); x_4 = lean_unsigned_to_nat(21u); -x_5 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__3; +x_5 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { if (lean_obj_tag(x_3) == 0) @@ -1429,8 +1428,8 @@ lean_object* x_12; lean_object* x_13; lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_12 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__4; -x_13 = l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__10(x_12, x_5, x_6, x_7); +x_12 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__4; +x_13 = l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9(x_12, x_5, x_6, x_7); return x_13; } default: @@ -1487,111 +1486,179 @@ lean_inc(x_21); x_24 = lean_apply_6(x_1, x_21, x_22, x_23, x_5, x_6, x_7); if (lean_obj_tag(x_24) == 0) { -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_25 = lean_ctor_get(x_24, 1); +lean_object* x_25; uint8_t x_26; +x_25 = lean_ctor_get(x_24, 0); lean_inc(x_25); +x_26 = lean_unbox(x_25); +lean_dec(x_25); +if (x_26 == 0) +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; +lean_dec(x_1); +x_27 = lean_ctor_get(x_24, 1); +lean_inc(x_27); lean_dec(x_24); -lean_inc(x_21); -x_26 = l_Lean_Elab_Info_updateContext_x3f(x_3, x_22); -x_27 = l_Lean_PersistentArray_toList___rarg(x_23); x_28 = lean_box(0); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_2); -x_29 = l_List_mapM_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11(x_1, x_2, x_26, x_27, x_28, x_5, x_6, x_25); +x_29 = lean_apply_7(x_2, x_21, x_22, x_23, x_28, x_5, x_6, x_27); if (lean_obj_tag(x_29) == 0) { -lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_30 = lean_ctor_get(x_29, 0); -lean_inc(x_30); -x_31 = lean_ctor_get(x_29, 1); -lean_inc(x_31); +uint8_t x_30; +x_30 = !lean_is_exclusive(x_29); +if (x_30 == 0) +{ +lean_object* x_31; +x_31 = lean_ctor_get(x_29, 0); +lean_ctor_set(x_3, 0, x_31); +lean_ctor_set(x_29, 0, x_3); +return x_29; +} +else +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_29, 0); +x_33 = lean_ctor_get(x_29, 1); +lean_inc(x_33); +lean_inc(x_32); lean_dec(x_29); -x_32 = lean_apply_7(x_2, x_21, x_22, x_23, x_30, x_5, x_6, x_31); -if (lean_obj_tag(x_32) == 0) +lean_ctor_set(x_3, 0, x_32); +x_34 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_34, 0, x_3); +lean_ctor_set(x_34, 1, x_33); +return x_34; +} +} +else { -uint8_t x_33; -x_33 = !lean_is_exclusive(x_32); -if (x_33 == 0) +uint8_t x_35; +lean_free_object(x_3); +x_35 = !lean_is_exclusive(x_29); +if (x_35 == 0) { -lean_object* x_34; lean_object* x_35; -x_34 = lean_ctor_get(x_32, 0); -x_35 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_35, 0, x_34); -lean_ctor_set(x_32, 0, x_35); -return x_32; +return x_29; } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_36 = lean_ctor_get(x_32, 0); -x_37 = lean_ctor_get(x_32, 1); +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_29, 0); +x_37 = lean_ctor_get(x_29, 1); lean_inc(x_37); lean_inc(x_36); -lean_dec(x_32); -x_38 = lean_alloc_ctor(1, 1, 0); +lean_dec(x_29); +x_38 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_38, 0, x_36); -x_39 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_39, 0, x_38); -lean_ctor_set(x_39, 1, x_37); -return x_39; +lean_ctor_set(x_38, 1, x_37); +return x_38; +} } } else { -uint8_t x_40; -x_40 = !lean_is_exclusive(x_32); -if (x_40 == 0) +lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_39 = lean_ctor_get(x_24, 1); +lean_inc(x_39); +lean_dec(x_24); +lean_inc(x_21); +x_40 = l_Lean_Elab_Info_updateContext_x3f(x_3, x_22); +x_41 = l_Lean_PersistentArray_toList___rarg(x_23); +x_42 = lean_box(0); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_2); +x_43 = l_List_mapM_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__10(x_1, x_2, x_40, x_41, x_42, x_5, x_6, x_39); +if (lean_obj_tag(x_43) == 0) { -return x_32; +lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_44 = lean_ctor_get(x_43, 0); +lean_inc(x_44); +x_45 = lean_ctor_get(x_43, 1); +lean_inc(x_45); +lean_dec(x_43); +x_46 = lean_apply_7(x_2, x_21, x_22, x_23, x_44, x_5, x_6, x_45); +if (lean_obj_tag(x_46) == 0) +{ +uint8_t x_47; +x_47 = !lean_is_exclusive(x_46); +if (x_47 == 0) +{ +lean_object* x_48; lean_object* x_49; +x_48 = lean_ctor_get(x_46, 0); +x_49 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_49, 0, x_48); +lean_ctor_set(x_46, 0, x_49); +return x_46; } else { -lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_ctor_get(x_32, 0); -x_42 = lean_ctor_get(x_32, 1); -lean_inc(x_42); -lean_inc(x_41); -lean_dec(x_32); -x_43 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_43, 0, x_41); -lean_ctor_set(x_43, 1, x_42); -return x_43; +lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_50 = lean_ctor_get(x_46, 0); +x_51 = lean_ctor_get(x_46, 1); +lean_inc(x_51); +lean_inc(x_50); +lean_dec(x_46); +x_52 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_52, 0, x_50); +x_53 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_53, 0, x_52); +lean_ctor_set(x_53, 1, x_51); +return x_53; +} +} +else +{ +uint8_t x_54; +x_54 = !lean_is_exclusive(x_46); +if (x_54 == 0) +{ +return x_46; +} +else +{ +lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_55 = lean_ctor_get(x_46, 0); +x_56 = lean_ctor_get(x_46, 1); +lean_inc(x_56); +lean_inc(x_55); +lean_dec(x_46); +x_57 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_57, 0, x_55); +lean_ctor_set(x_57, 1, x_56); +return x_57; } } } else { -uint8_t x_44; +uint8_t x_58; lean_dec(x_23); lean_dec(x_22); lean_dec(x_21); lean_dec(x_6); lean_dec(x_5); lean_dec(x_2); -x_44 = !lean_is_exclusive(x_29); -if (x_44 == 0) +x_58 = !lean_is_exclusive(x_43); +if (x_58 == 0) { -return x_29; +return x_43; } else { -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_29, 0); -x_46 = lean_ctor_get(x_29, 1); -lean_inc(x_46); -lean_inc(x_45); -lean_dec(x_29); -x_47 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_47, 0, x_45); -lean_ctor_set(x_47, 1, x_46); -return x_47; +lean_object* x_59; lean_object* x_60; lean_object* x_61; +x_59 = lean_ctor_get(x_43, 0); +x_60 = lean_ctor_get(x_43, 1); +lean_inc(x_60); +lean_inc(x_59); +lean_dec(x_43); +x_61 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_61, 0, x_59); +lean_ctor_set(x_61, 1, x_60); +return x_61; +} } } } else { -uint8_t x_48; +uint8_t x_62; lean_dec(x_23); lean_dec(x_22); lean_free_object(x_3); @@ -1600,210 +1667,269 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_2); lean_dec(x_1); -x_48 = !lean_is_exclusive(x_24); -if (x_48 == 0) +x_62 = !lean_is_exclusive(x_24); +if (x_62 == 0) { return x_24; } else { -lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_49 = lean_ctor_get(x_24, 0); -x_50 = lean_ctor_get(x_24, 1); -lean_inc(x_50); -lean_inc(x_49); +lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_63 = lean_ctor_get(x_24, 0); +x_64 = lean_ctor_get(x_24, 1); +lean_inc(x_64); +lean_inc(x_63); lean_dec(x_24); -x_51 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_51, 0, x_49); -lean_ctor_set(x_51, 1, x_50); -return x_51; +x_65 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_65, 0, x_63); +lean_ctor_set(x_65, 1, x_64); +return x_65; } } } else { -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_52 = lean_ctor_get(x_3, 0); -lean_inc(x_52); +lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; +x_66 = lean_ctor_get(x_3, 0); +lean_inc(x_66); lean_dec(x_3); -x_53 = lean_ctor_get(x_4, 0); -lean_inc(x_53); -x_54 = lean_ctor_get(x_4, 1); -lean_inc(x_54); +x_67 = lean_ctor_get(x_4, 0); +lean_inc(x_67); +x_68 = lean_ctor_get(x_4, 1); +lean_inc(x_68); lean_dec(x_4); lean_inc(x_1); lean_inc(x_6); lean_inc(x_5); -lean_inc(x_54); -lean_inc(x_53); -lean_inc(x_52); -x_55 = lean_apply_6(x_1, x_52, x_53, x_54, x_5, x_6, x_7); -if (lean_obj_tag(x_55) == 0) +lean_inc(x_68); +lean_inc(x_67); +lean_inc(x_66); +x_69 = lean_apply_6(x_1, x_66, x_67, x_68, x_5, x_6, x_7); +if (lean_obj_tag(x_69) == 0) { -lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; -x_56 = lean_ctor_get(x_55, 1); -lean_inc(x_56); -lean_dec(x_55); -lean_inc(x_52); -x_57 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_57, 0, x_52); -x_58 = l_Lean_Elab_Info_updateContext_x3f(x_57, x_53); -x_59 = l_Lean_PersistentArray_toList___rarg(x_54); -x_60 = lean_box(0); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_2); -x_61 = l_List_mapM_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11(x_1, x_2, x_58, x_59, x_60, x_5, x_6, x_56); -if (lean_obj_tag(x_61) == 0) +lean_object* x_70; uint8_t x_71; +x_70 = lean_ctor_get(x_69, 0); +lean_inc(x_70); +x_71 = lean_unbox(x_70); +lean_dec(x_70); +if (x_71 == 0) { -lean_object* x_62; lean_object* x_63; lean_object* x_64; -x_62 = lean_ctor_get(x_61, 0); -lean_inc(x_62); -x_63 = lean_ctor_get(x_61, 1); -lean_inc(x_63); -lean_dec(x_61); -x_64 = lean_apply_7(x_2, x_52, x_53, x_54, x_62, x_5, x_6, x_63); -if (lean_obj_tag(x_64) == 0) +lean_object* x_72; lean_object* x_73; lean_object* x_74; +lean_dec(x_1); +x_72 = lean_ctor_get(x_69, 1); +lean_inc(x_72); +lean_dec(x_69); +x_73 = lean_box(0); +x_74 = lean_apply_7(x_2, x_66, x_67, x_68, x_73, x_5, x_6, x_72); +if (lean_obj_tag(x_74) == 0) { -lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_65 = lean_ctor_get(x_64, 0); -lean_inc(x_65); -x_66 = lean_ctor_get(x_64, 1); +lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; +x_75 = lean_ctor_get(x_74, 0); +lean_inc(x_75); +x_76 = lean_ctor_get(x_74, 1); +lean_inc(x_76); +if (lean_is_exclusive(x_74)) { + lean_ctor_release(x_74, 0); + lean_ctor_release(x_74, 1); + x_77 = x_74; +} else { + lean_dec_ref(x_74); + x_77 = lean_box(0); +} +x_78 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_78, 0, x_75); +if (lean_is_scalar(x_77)) { + x_79 = lean_alloc_ctor(0, 2, 0); +} else { + x_79 = x_77; +} +lean_ctor_set(x_79, 0, x_78); +lean_ctor_set(x_79, 1, x_76); +return x_79; +} +else +{ +lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; +x_80 = lean_ctor_get(x_74, 0); +lean_inc(x_80); +x_81 = lean_ctor_get(x_74, 1); +lean_inc(x_81); +if (lean_is_exclusive(x_74)) { + lean_ctor_release(x_74, 0); + lean_ctor_release(x_74, 1); + x_82 = x_74; +} else { + lean_dec_ref(x_74); + x_82 = lean_box(0); +} +if (lean_is_scalar(x_82)) { + x_83 = lean_alloc_ctor(1, 2, 0); +} else { + x_83 = x_82; +} +lean_ctor_set(x_83, 0, x_80); +lean_ctor_set(x_83, 1, x_81); +return x_83; +} +} +else +{ +lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; +x_84 = lean_ctor_get(x_69, 1); +lean_inc(x_84); +lean_dec(x_69); lean_inc(x_66); -if (lean_is_exclusive(x_64)) { - lean_ctor_release(x_64, 0); - lean_ctor_release(x_64, 1); - x_67 = x_64; +x_85 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_85, 0, x_66); +x_86 = l_Lean_Elab_Info_updateContext_x3f(x_85, x_67); +x_87 = l_Lean_PersistentArray_toList___rarg(x_68); +x_88 = lean_box(0); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_2); +x_89 = l_List_mapM_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__10(x_1, x_2, x_86, x_87, x_88, x_5, x_6, x_84); +if (lean_obj_tag(x_89) == 0) +{ +lean_object* x_90; lean_object* x_91; lean_object* x_92; +x_90 = lean_ctor_get(x_89, 0); +lean_inc(x_90); +x_91 = lean_ctor_get(x_89, 1); +lean_inc(x_91); +lean_dec(x_89); +x_92 = lean_apply_7(x_2, x_66, x_67, x_68, x_90, x_5, x_6, x_91); +if (lean_obj_tag(x_92) == 0) +{ +lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; +x_93 = lean_ctor_get(x_92, 0); +lean_inc(x_93); +x_94 = lean_ctor_get(x_92, 1); +lean_inc(x_94); +if (lean_is_exclusive(x_92)) { + lean_ctor_release(x_92, 0); + lean_ctor_release(x_92, 1); + x_95 = x_92; } else { - lean_dec_ref(x_64); - x_67 = lean_box(0); + lean_dec_ref(x_92); + x_95 = lean_box(0); } -x_68 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_68, 0, x_65); -if (lean_is_scalar(x_67)) { - x_69 = lean_alloc_ctor(0, 2, 0); +x_96 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_96, 0, x_93); +if (lean_is_scalar(x_95)) { + x_97 = lean_alloc_ctor(0, 2, 0); } else { - x_69 = x_67; + x_97 = x_95; } -lean_ctor_set(x_69, 0, x_68); -lean_ctor_set(x_69, 1, x_66); -return x_69; +lean_ctor_set(x_97, 0, x_96); +lean_ctor_set(x_97, 1, x_94); +return x_97; } else { -lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_70 = lean_ctor_get(x_64, 0); -lean_inc(x_70); -x_71 = lean_ctor_get(x_64, 1); -lean_inc(x_71); -if (lean_is_exclusive(x_64)) { - lean_ctor_release(x_64, 0); - lean_ctor_release(x_64, 1); - x_72 = x_64; +lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; +x_98 = lean_ctor_get(x_92, 0); +lean_inc(x_98); +x_99 = lean_ctor_get(x_92, 1); +lean_inc(x_99); +if (lean_is_exclusive(x_92)) { + lean_ctor_release(x_92, 0); + lean_ctor_release(x_92, 1); + x_100 = x_92; } else { - lean_dec_ref(x_64); - x_72 = lean_box(0); + lean_dec_ref(x_92); + x_100 = lean_box(0); } -if (lean_is_scalar(x_72)) { - x_73 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_100)) { + x_101 = lean_alloc_ctor(1, 2, 0); } else { - x_73 = x_72; + x_101 = x_100; } -lean_ctor_set(x_73, 0, x_70); -lean_ctor_set(x_73, 1, x_71); -return x_73; +lean_ctor_set(x_101, 0, x_98); +lean_ctor_set(x_101, 1, x_99); +return x_101; } } else { -lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; -lean_dec(x_54); -lean_dec(x_53); -lean_dec(x_52); +lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; +lean_dec(x_68); +lean_dec(x_67); +lean_dec(x_66); lean_dec(x_6); lean_dec(x_5); lean_dec(x_2); -x_74 = lean_ctor_get(x_61, 0); -lean_inc(x_74); -x_75 = lean_ctor_get(x_61, 1); -lean_inc(x_75); -if (lean_is_exclusive(x_61)) { - lean_ctor_release(x_61, 0); - lean_ctor_release(x_61, 1); - x_76 = x_61; +x_102 = lean_ctor_get(x_89, 0); +lean_inc(x_102); +x_103 = lean_ctor_get(x_89, 1); +lean_inc(x_103); +if (lean_is_exclusive(x_89)) { + lean_ctor_release(x_89, 0); + lean_ctor_release(x_89, 1); + x_104 = x_89; } else { - lean_dec_ref(x_61); - x_76 = lean_box(0); + lean_dec_ref(x_89); + x_104 = lean_box(0); } -if (lean_is_scalar(x_76)) { - x_77 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_104)) { + x_105 = lean_alloc_ctor(1, 2, 0); } else { - x_77 = x_76; + x_105 = x_104; +} +lean_ctor_set(x_105, 0, x_102); +lean_ctor_set(x_105, 1, x_103); +return x_105; } -lean_ctor_set(x_77, 0, x_74); -lean_ctor_set(x_77, 1, x_75); -return x_77; } } else { -lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; -lean_dec(x_54); -lean_dec(x_53); -lean_dec(x_52); +lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; +lean_dec(x_68); +lean_dec(x_67); +lean_dec(x_66); lean_dec(x_6); lean_dec(x_5); lean_dec(x_2); lean_dec(x_1); -x_78 = lean_ctor_get(x_55, 0); -lean_inc(x_78); -x_79 = lean_ctor_get(x_55, 1); -lean_inc(x_79); -if (lean_is_exclusive(x_55)) { - lean_ctor_release(x_55, 0); - lean_ctor_release(x_55, 1); - x_80 = x_55; +x_106 = lean_ctor_get(x_69, 0); +lean_inc(x_106); +x_107 = lean_ctor_get(x_69, 1); +lean_inc(x_107); +if (lean_is_exclusive(x_69)) { + lean_ctor_release(x_69, 0); + lean_ctor_release(x_69, 1); + x_108 = x_69; } else { - lean_dec_ref(x_55); - x_80 = lean_box(0); + lean_dec_ref(x_69); + x_108 = lean_box(0); } -if (lean_is_scalar(x_80)) { - x_81 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_108)) { + x_109 = lean_alloc_ctor(1, 2, 0); } else { - x_81 = x_80; + x_109 = x_108; } -lean_ctor_set(x_81, 0, x_78); -lean_ctor_set(x_81, 1, x_79); -return x_81; +lean_ctor_set(x_109, 0, x_106); +lean_ctor_set(x_109, 1, x_107); +return x_109; } } } default: { -lean_object* x_82; lean_object* x_83; +lean_object* x_110; lean_object* x_111; lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_82 = lean_box(0); -x_83 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_83, 0, x_82); -lean_ctor_set(x_83, 1, x_7); -return x_83; -} -} +x_110 = lean_box(0); +x_111 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_111, 0, x_110); +lean_ctor_set(x_111, 1, x_7); +return x_111; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -lean_object* x_7; lean_object* x_8; -x_7 = lean_box(0); -x_8 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9(x_1, x_2, x_7, x_3, x_4, x_5, x_6); -return x_8; } } LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__7___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { @@ -1814,64 +1940,76 @@ x_9 = lean_apply_6(x_1, x_2, x_3, x_4, x_6, x_7, x_8); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { -lean_object* x_7; lean_object* x_8; -x_7 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__7___lambda__1___boxed), 8, 1); -lean_closure_set(x_7, 0, x_2); -x_8 = l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8(x_1, x_7, x_3, x_4, x_5, x_6); -if (lean_obj_tag(x_8) == 0) +lean_object* x_8; lean_object* x_9; +x_8 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__7___lambda__1___boxed), 8, 1); +lean_closure_set(x_8, 0, x_2); +x_9 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8(x_1, x_8, x_3, x_4, x_5, x_6, x_7); +if (lean_obj_tag(x_9) == 0) { -uint8_t x_9; -x_9 = !lean_is_exclusive(x_8); -if (x_9 == 0) +uint8_t x_10; +x_10 = !lean_is_exclusive(x_9); +if (x_10 == 0) { -lean_object* x_10; lean_object* x_11; -x_10 = lean_ctor_get(x_8, 0); -lean_dec(x_10); -x_11 = lean_box(0); -lean_ctor_set(x_8, 0, x_11); -return x_8; +lean_object* x_11; lean_object* x_12; +x_11 = lean_ctor_get(x_9, 0); +lean_dec(x_11); +x_12 = lean_box(0); +lean_ctor_set(x_9, 0, x_12); +return x_9; } else { -lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_12 = lean_ctor_get(x_8, 1); -lean_inc(x_12); -lean_dec(x_8); -x_13 = lean_box(0); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_13); -lean_ctor_set(x_14, 1, x_12); -return x_14; +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_9, 1); +lean_inc(x_13); +lean_dec(x_9); +x_14 = lean_box(0); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_13); +return x_15; } } else { -uint8_t x_15; -x_15 = !lean_is_exclusive(x_8); -if (x_15 == 0) +uint8_t x_16; +x_16 = !lean_is_exclusive(x_9); +if (x_16 == 0) { -return x_8; +return x_9; } else { -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_8, 0); -x_17 = lean_ctor_get(x_8, 1); +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_9, 0); +x_18 = lean_ctor_get(x_9, 1); +lean_inc(x_18); lean_inc(x_17); -lean_inc(x_16); -lean_dec(x_8); -x_18 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_18, 0, x_16); -lean_ctor_set(x_18, 1, x_17); -return x_18; +lean_dec(x_9); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set(x_19, 1, x_18); +return x_19; +} +} } } +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +uint8_t x_7; lean_object* x_8; lean_object* x_9; +x_7 = 1; +x_8 = lean_box(x_7); +x_9 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_9, 0, x_8); +lean_ctor_set(x_9, 1, x_6); +return x_9; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; @@ -1885,11 +2023,11 @@ x_10 = lean_whnf(x_8, x_2, x_3, x_4, x_5, x_9); return x_10; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; -x_13 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__1), 6, 1); +x_13 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__2), 6, 1); lean_closure_set(x_13, 0, x_9); x_14 = l_Lean_Elab_TermInfo_runMetaM___rarg(x_1, x_2, x_13, x_12); if (lean_obj_tag(x_14) == 0) @@ -2248,7 +2386,7 @@ return x_92; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { lean_object* x_12; @@ -2281,7 +2419,7 @@ lean_inc(x_18); x_19 = lean_ctor_get(x_17, 1); lean_inc(x_19); lean_dec(x_17); -x_20 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__2(x_2, x_3, x_4, x_5, x_6, x_1, x_12, x_15, x_18, x_9, x_10, x_19); +x_20 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__3(x_2, x_3, x_4, x_5, x_6, x_1, x_12, x_15, x_18, x_9, x_10, x_19); lean_dec(x_15); return x_20; } @@ -2345,7 +2483,7 @@ lean_inc(x_36); x_37 = lean_ctor_get(x_14, 0); lean_inc(x_37); lean_dec(x_14); -x_38 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__2(x_2, x_3, x_4, x_5, x_6, x_1, x_12, x_36, x_37, x_9, x_10, x_11); +x_38 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__3(x_2, x_3, x_4, x_5, x_6, x_1, x_12, x_36, x_37, x_9, x_10, x_11); lean_dec(x_36); return x_38; } @@ -2386,7 +2524,7 @@ return x_42; } } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__4___closed__1() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__5___closed__1() { _start: { lean_object* x_1; @@ -2394,7 +2532,7 @@ x_1 = l_Lean_Linter_linter_constructorNameAsVariable; return x_1; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; @@ -2403,7 +2541,7 @@ lean_inc(x_12); x_13 = lean_ctor_get(x_12, 3); lean_inc(x_13); lean_dec(x_12); -x_14 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__4___closed__1; +x_14 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__5___closed__1; x_15 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_13, x_14); lean_dec(x_13); if (x_15 == 0) @@ -2425,12 +2563,12 @@ else { lean_object* x_18; lean_object* x_19; x_18 = lean_box(0); -x_19 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__3(x_2, x_3, x_1, x_4, x_5, x_6, x_7, x_18, x_9, x_10, x_11); +x_19 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__4(x_2, x_3, x_1, x_4, x_5, x_6, x_7, x_18, x_9, x_10, x_11); return x_19; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { lean_object* x_14; lean_object* x_15; @@ -2516,7 +2654,7 @@ if (x_30 == 0) { lean_object* x_31; lean_object* x_32; x_31 = lean_box(0); -x_32 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__4(x_4, x_14, x_2, x_5, x_6, x_7, x_8, x_31, x_11, x_12, x_13); +x_32 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__5(x_4, x_14, x_2, x_5, x_6, x_7, x_8, x_31, x_11, x_12, x_13); return x_32; } else @@ -2557,7 +2695,7 @@ return x_36; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { if (lean_obj_tag(x_5) == 1) @@ -2627,7 +2765,7 @@ if (x_36 == 0) lean_object* x_37; lean_object* x_38; lean_free_object(x_17); x_37 = lean_box(0); -x_38 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__5(x_5, x_10, x_12, x_4, x_2, x_1, x_16, x_11, x_3, x_37, x_7, x_8, x_20); +x_38 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__6(x_5, x_10, x_12, x_4, x_2, x_1, x_16, x_11, x_3, x_37, x_7, x_8, x_20); lean_dec(x_5); return x_38; } @@ -2679,7 +2817,7 @@ if (x_57 == 0) { lean_object* x_58; lean_object* x_59; x_58 = lean_box(0); -x_59 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__5(x_5, x_10, x_12, x_4, x_2, x_1, x_16, x_11, x_3, x_58, x_7, x_8, x_41); +x_59 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__6(x_5, x_10, x_12, x_4, x_2, x_1, x_16, x_11, x_3, x_58, x_7, x_8, x_41); lean_dec(x_5); return x_59; } @@ -2731,26 +2869,15 @@ return x_65; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -lean_object* x_7; lean_object* x_8; -x_7 = lean_box(0); -x_8 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_8, 0, x_7); -lean_ctor_set(x_8, 1, x_6); -return x_8; -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___closed__1() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__7___boxed), 6, 0); +x_1 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__1___boxed), 6, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { uint8_t x_11; @@ -2770,65 +2897,66 @@ return x_12; } else { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_dec(x_7); x_13 = lean_array_uget(x_4, x_6); lean_inc(x_1); lean_inc(x_2); lean_inc(x_3); -x_14 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__6___boxed), 9, 3); +x_14 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__7___boxed), 9, 3); lean_closure_set(x_14, 0, x_3); lean_closure_set(x_14, 1, x_2); lean_closure_set(x_14, 2, x_1); -x_15 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___closed__1; +x_15 = lean_box(0); +x_16 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___closed__1; lean_inc(x_9); lean_inc(x_8); -x_16 = l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__7(x_14, x_15, x_13, x_8, x_9, x_10); -if (lean_obj_tag(x_16) == 0) +x_17 = l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__7(x_16, x_14, x_15, x_13, x_8, x_9, x_10); +if (lean_obj_tag(x_17) == 0) { -lean_object* x_17; size_t x_18; size_t x_19; lean_object* x_20; -x_17 = lean_ctor_get(x_16, 1); -lean_inc(x_17); -lean_dec(x_16); -x_18 = 1; -x_19 = lean_usize_add(x_6, x_18); -x_20 = lean_box(0); -x_6 = x_19; -x_7 = x_20; -x_10 = x_17; +lean_object* x_18; size_t x_19; size_t x_20; lean_object* x_21; +x_18 = lean_ctor_get(x_17, 1); +lean_inc(x_18); +lean_dec(x_17); +x_19 = 1; +x_20 = lean_usize_add(x_6, x_19); +x_21 = lean_box(0); +x_6 = x_20; +x_7 = x_21; +x_10 = x_18; goto _start; } else { -uint8_t x_22; +uint8_t x_23; lean_dec(x_9); lean_dec(x_8); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_22 = !lean_is_exclusive(x_16); -if (x_22 == 0) +x_23 = !lean_is_exclusive(x_17); +if (x_23 == 0) { -return x_16; +return x_17; } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_16, 0); -x_24 = lean_ctor_get(x_16, 1); +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_17, 0); +x_25 = lean_ctor_get(x_17, 1); +lean_inc(x_25); lean_inc(x_24); -lean_inc(x_23); -lean_dec(x_16); -x_25 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_25, 0, x_23); -lean_ctor_set(x_25, 1, x_24); -return x_25; +lean_dec(x_17); +x_26 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_26, 0, x_24); +lean_ctor_set(x_26, 1, x_25); +return x_26; } } } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -2853,7 +2981,7 @@ goto _start; } } } -static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__1() { +static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__1() { _start: { lean_object* x_1; @@ -2861,16 +2989,16 @@ x_1 = lean_mk_string_unchecked("note: this linter can be disabled with `set_opti return x_1; } } -static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__2() { +static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__1; +x_1 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__3() { +static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__3() { _start: { lean_object* x_1; @@ -2878,16 +3006,16 @@ x_1 = lean_mk_string_unchecked(" false`", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__4() { +static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__3; +x_1 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__3; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__5() { +static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__5() { _start: { lean_object* x_1; lean_object* x_2; @@ -2896,7 +3024,7 @@ x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__6() { +static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__6() { _start: { lean_object* x_1; @@ -2904,16 +3032,16 @@ x_1 = lean_mk_string_unchecked("\n", 1, 1); return x_1; } } -static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__7() { +static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__7() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__6; +x_1 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__6; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { uint8_t x_7; @@ -2926,19 +3054,19 @@ x_9 = lean_ctor_get(x_1, 1); lean_dec(x_9); lean_inc(x_8); x_10 = l_Lean_MessageData_ofName(x_8); -x_11 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__2; +x_11 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__2; lean_ctor_set_tag(x_1, 7); lean_ctor_set(x_1, 1, x_10); lean_ctor_set(x_1, 0, x_11); -x_12 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__4; +x_12 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__4; x_13 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_13, 0, x_1); lean_ctor_set(x_13, 1, x_12); -x_14 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__5; +x_14 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__5; x_15 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_15, 0, x_14); lean_ctor_set(x_15, 1, x_3); -x_16 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__7; +x_16 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__7; x_17 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_17, 0, x_15); lean_ctor_set(x_17, 1, x_16); @@ -2963,19 +3091,19 @@ lean_inc(x_23); lean_dec(x_1); lean_inc(x_23); x_24 = l_Lean_MessageData_ofName(x_23); -x_25 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__2; +x_25 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__2; x_26 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_26, 0, x_25); lean_ctor_set(x_26, 1, x_24); -x_27 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__4; +x_27 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__4; x_28 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_28, 0, x_26); lean_ctor_set(x_28, 1, x_27); -x_29 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__5; +x_29 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__5; x_30 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_30, 0, x_29); lean_ctor_set(x_30, 1, x_3); -x_31 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__7; +x_31 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__7; x_32 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_32, 0, x_30); lean_ctor_set(x_32, 1, x_31); @@ -2994,7 +3122,7 @@ return x_37; } } } -LEAN_EXPORT uint8_t l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___lambda__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___lambda__1(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; uint8_t x_7; @@ -3006,15 +3134,15 @@ x_7 = lean_nat_dec_lt(x_4, x_6); return x_7; } } -static lean_object* _init_l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__1() { +static lean_object* _init_l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___lambda__1___boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___lambda__1___boxed), 2, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -3027,7 +3155,7 @@ return x_1; else { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; -x_5 = l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__1; +x_5 = l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__1; lean_inc(x_2); x_6 = l_Array_qpartition___rarg(x_1, x_5, x_2, x_3); x_7 = lean_ctor_get(x_6, 0); @@ -3039,7 +3167,7 @@ x_9 = lean_nat_dec_le(x_3, x_7); if (x_9 == 0) { lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_10 = l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15(x_8, x_2, x_7); +x_10 = l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14(x_8, x_2, x_7); x_11 = lean_unsigned_to_nat(1u); x_12 = lean_nat_add(x_7, x_11); lean_dec(x_7); @@ -3056,7 +3184,7 @@ return x_8; } } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__1() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__1() { _start: { lean_object* x_1; @@ -3064,16 +3192,16 @@ x_1 = lean_mk_string_unchecked("Local variable '", 16, 16); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__2() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__1; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__3() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__3() { _start: { lean_object* x_1; @@ -3081,16 +3209,16 @@ x_1 = lean_mk_string_unchecked("' resembles constructor '", 25, 25); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__4() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__3; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__3; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__5() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__5() { _start: { lean_object* x_1; @@ -3098,16 +3226,16 @@ x_1 = lean_mk_string_unchecked("' - ", 4, 4); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__6() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__6() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__5; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__5; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__7() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__7() { _start: { lean_object* x_1; @@ -3115,16 +3243,16 @@ x_1 = lean_mk_string_unchecked("write '.", 8, 8); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__8() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__8() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__7; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__7; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__9() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__9() { _start: { lean_object* x_1; @@ -3132,16 +3260,16 @@ x_1 = lean_mk_string_unchecked("' (with a dot) or '", 19, 19); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__10() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__10() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__9; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__9; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__11() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__11() { _start: { lean_object* x_1; @@ -3149,16 +3277,16 @@ x_1 = lean_mk_string_unchecked("' to use the constructor.", 25, 25); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__12() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__12() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__11; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__11; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { uint8_t x_8; @@ -3197,12 +3325,12 @@ x_17 = lean_ctor_get(x_12, 0); x_18 = lean_ctor_get(x_15, 0); x_19 = lean_ctor_get(x_15, 1); x_20 = l_Lean_MessageData_ofName(x_18); -x_21 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__2; +x_21 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__2; lean_inc(x_20); lean_ctor_set_tag(x_15, 7); lean_ctor_set(x_15, 1, x_20); lean_ctor_set(x_15, 0, x_21); -x_22 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__4; +x_22 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__4; lean_ctor_set_tag(x_12, 7); lean_ctor_set(x_12, 1, x_22); lean_ctor_set(x_12, 0, x_15); @@ -3211,31 +3339,31 @@ lean_inc(x_23); lean_ctor_set_tag(x_10, 7); lean_ctor_set(x_10, 1, x_23); lean_ctor_set(x_10, 0, x_12); -x_24 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__6; +x_24 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__6; x_25 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_25, 0, x_10); lean_ctor_set(x_25, 1, x_24); -x_26 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__8; +x_26 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__8; x_27 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_27, 0, x_26); lean_ctor_set(x_27, 1, x_20); -x_28 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__10; +x_28 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__10; x_29 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_29, 0, x_27); lean_ctor_set(x_29, 1, x_28); x_30 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_30, 0, x_29); lean_ctor_set(x_30, 1, x_23); -x_31 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__12; +x_31 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__12; x_32 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_32, 0, x_30); lean_ctor_set(x_32, 1, x_31); x_33 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_33, 0, x_25); lean_ctor_set(x_33, 1, x_32); -x_34 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__4___closed__1; +x_34 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__5___closed__1; lean_inc(x_5); -x_35 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14(x_34, x_17, x_33, x_5, x_6, x_7); +x_35 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13(x_34, x_17, x_33, x_5, x_6, x_7); lean_dec(x_17); x_36 = lean_ctor_get(x_35, 1); lean_inc(x_36); @@ -3258,12 +3386,12 @@ lean_inc(x_43); lean_inc(x_42); lean_dec(x_15); x_44 = l_Lean_MessageData_ofName(x_42); -x_45 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__2; +x_45 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__2; lean_inc(x_44); x_46 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_46, 0, x_45); lean_ctor_set(x_46, 1, x_44); -x_47 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__4; +x_47 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__4; lean_ctor_set_tag(x_12, 7); lean_ctor_set(x_12, 1, x_47); lean_ctor_set(x_12, 0, x_46); @@ -3272,31 +3400,31 @@ lean_inc(x_48); lean_ctor_set_tag(x_10, 7); lean_ctor_set(x_10, 1, x_48); lean_ctor_set(x_10, 0, x_12); -x_49 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__6; +x_49 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__6; x_50 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_50, 0, x_10); lean_ctor_set(x_50, 1, x_49); -x_51 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__8; +x_51 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__8; x_52 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_52, 0, x_51); lean_ctor_set(x_52, 1, x_44); -x_53 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__10; +x_53 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__10; x_54 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_54, 0, x_52); lean_ctor_set(x_54, 1, x_53); x_55 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_55, 0, x_54); lean_ctor_set(x_55, 1, x_48); -x_56 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__12; +x_56 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__12; x_57 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_57, 0, x_55); lean_ctor_set(x_57, 1, x_56); x_58 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_58, 0, x_50); lean_ctor_set(x_58, 1, x_57); -x_59 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__4___closed__1; +x_59 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__5___closed__1; lean_inc(x_5); -x_60 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14(x_59, x_41, x_58, x_5, x_6, x_7); +x_60 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13(x_59, x_41, x_58, x_5, x_6, x_7); lean_dec(x_41); x_61 = lean_ctor_get(x_60, 1); lean_inc(x_61); @@ -3331,7 +3459,7 @@ if (lean_is_exclusive(x_66)) { x_70 = lean_box(0); } x_71 = l_Lean_MessageData_ofName(x_68); -x_72 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__2; +x_72 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__2; lean_inc(x_71); if (lean_is_scalar(x_70)) { x_73 = lean_alloc_ctor(7, 2, 0); @@ -3341,7 +3469,7 @@ if (lean_is_scalar(x_70)) { } lean_ctor_set(x_73, 0, x_72); lean_ctor_set(x_73, 1, x_71); -x_74 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__4; +x_74 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__4; x_75 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_75, 0, x_73); lean_ctor_set(x_75, 1, x_74); @@ -3350,31 +3478,31 @@ lean_inc(x_76); lean_ctor_set_tag(x_10, 7); lean_ctor_set(x_10, 1, x_76); lean_ctor_set(x_10, 0, x_75); -x_77 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__6; +x_77 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__6; x_78 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_78, 0, x_10); lean_ctor_set(x_78, 1, x_77); -x_79 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__8; +x_79 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__8; x_80 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_80, 0, x_79); lean_ctor_set(x_80, 1, x_71); -x_81 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__10; +x_81 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__10; x_82 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_82, 0, x_80); lean_ctor_set(x_82, 1, x_81); x_83 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_83, 0, x_82); lean_ctor_set(x_83, 1, x_76); -x_84 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__12; +x_84 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__12; x_85 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_85, 0, x_83); lean_ctor_set(x_85, 1, x_84); x_86 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_86, 0, x_78); lean_ctor_set(x_86, 1, x_85); -x_87 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__4___closed__1; +x_87 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__5___closed__1; lean_inc(x_5); -x_88 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14(x_87, x_67, x_86, x_5, x_6, x_7); +x_88 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13(x_87, x_67, x_86, x_5, x_6, x_7); lean_dec(x_67); x_89 = lean_ctor_get(x_88, 1); lean_inc(x_89); @@ -3419,7 +3547,7 @@ if (lean_is_exclusive(x_95)) { x_100 = lean_box(0); } x_101 = l_Lean_MessageData_ofName(x_98); -x_102 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__2; +x_102 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__2; lean_inc(x_101); if (lean_is_scalar(x_100)) { x_103 = lean_alloc_ctor(7, 2, 0); @@ -3429,7 +3557,7 @@ if (lean_is_scalar(x_100)) { } lean_ctor_set(x_103, 0, x_102); lean_ctor_set(x_103, 1, x_101); -x_104 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__4; +x_104 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__4; if (lean_is_scalar(x_97)) { x_105 = lean_alloc_ctor(7, 2, 0); } else { @@ -3443,31 +3571,31 @@ lean_inc(x_106); x_107 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_107, 0, x_105); lean_ctor_set(x_107, 1, x_106); -x_108 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__6; +x_108 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__6; x_109 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_109, 0, x_107); lean_ctor_set(x_109, 1, x_108); -x_110 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__8; +x_110 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__8; x_111 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_111, 0, x_110); lean_ctor_set(x_111, 1, x_101); -x_112 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__10; +x_112 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__10; x_113 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_113, 0, x_111); lean_ctor_set(x_113, 1, x_112); x_114 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_114, 0, x_113); lean_ctor_set(x_114, 1, x_106); -x_115 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__12; +x_115 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__12; x_116 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_116, 0, x_114); lean_ctor_set(x_116, 1, x_115); x_117 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_117, 0, x_109); lean_ctor_set(x_117, 1, x_116); -x_118 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__4___closed__1; +x_118 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__5___closed__1; lean_inc(x_5); -x_119 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14(x_118, x_96, x_117, x_5, x_6, x_7); +x_119 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13(x_118, x_96, x_117, x_5, x_6, x_7); lean_dec(x_96); x_120 = lean_ctor_get(x_119, 1); lean_inc(x_120); @@ -3483,7 +3611,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__17(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { uint8_t x_5; @@ -3492,7 +3620,7 @@ if (x_5 == 0) { lean_object* x_6; lean_object* x_7; size_t x_8; size_t x_9; x_6 = lean_array_uget(x_1, x_2); -x_7 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13(x_4, x_6); +x_7 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12(x_4, x_6); lean_dec(x_6); x_8 = 1; x_9 = lean_usize_add(x_2, x_8); @@ -3617,7 +3745,7 @@ x_23 = lean_box(0); lean_inc(x_3); lean_inc(x_2); lean_inc(x_19); -x_24 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12(x_9, x_16, x_19, x_15, x_21, x_22, x_23, x_2, x_3, x_20); +x_24 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11(x_9, x_16, x_19, x_15, x_21, x_22, x_23, x_2, x_3, x_20); lean_dec(x_15); if (lean_obj_tag(x_24) == 0) { @@ -3645,9 +3773,9 @@ lean_dec(x_30); lean_dec(x_29); x_33 = l_Lean_Linter_constructorNameAsVariable___elambda__1___closed__4; x_34 = l_Lean_Linter_constructorNameAsVariable___elambda__1___closed__6; -x_35 = l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15(x_33, x_31, x_34); +x_35 = l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14(x_33, x_31, x_34); x_36 = lean_array_size(x_35); -x_37 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16(x_35, x_36, x_22, x_23, x_2, x_3, x_28); +x_37 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15(x_35, x_36, x_22, x_23, x_2, x_3, x_28); lean_dec(x_3); lean_dec(x_35); x_38 = !lean_is_exclusive(x_37); @@ -3682,9 +3810,9 @@ lean_dec(x_30); lean_dec(x_29); x_43 = l_Lean_Linter_constructorNameAsVariable___elambda__1___closed__4; x_44 = l_Lean_Linter_constructorNameAsVariable___elambda__1___closed__6; -x_45 = l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15(x_43, x_31, x_44); +x_45 = l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14(x_43, x_31, x_44); x_46 = lean_array_size(x_45); -x_47 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16(x_45, x_46, x_22, x_23, x_2, x_3, x_28); +x_47 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15(x_45, x_46, x_22, x_23, x_2, x_3, x_28); lean_dec(x_3); lean_dec(x_45); x_48 = !lean_is_exclusive(x_47); @@ -3714,16 +3842,16 @@ size_t x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_objec x_52 = lean_usize_of_nat(x_30); lean_dec(x_30); x_53 = l_Lean_Linter_constructorNameAsVariable___elambda__1___closed__4; -x_54 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__17(x_29, x_22, x_52, x_53); +x_54 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16(x_29, x_22, x_52, x_53); lean_dec(x_29); x_55 = lean_array_get_size(x_54); x_56 = lean_unsigned_to_nat(1u); x_57 = lean_nat_sub(x_55, x_56); lean_dec(x_55); -x_58 = l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15(x_54, x_31, x_57); +x_58 = l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14(x_54, x_31, x_57); lean_dec(x_57); x_59 = lean_array_size(x_58); -x_60 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16(x_58, x_59, x_22, x_23, x_2, x_3, x_28); +x_60 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15(x_58, x_59, x_22, x_23, x_2, x_3, x_28); lean_dec(x_3); lean_dec(x_58); x_61 = !lean_is_exclusive(x_60); @@ -3861,11 +3989,24 @@ lean_dec(x_5); return x_9; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; +x_7 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; -x_13 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_13 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_8); @@ -3873,11 +4014,11 @@ lean_dec(x_4); return x_13; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { lean_object* x_12; -x_12 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_12 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -3885,11 +4026,11 @@ lean_dec(x_5); return x_12; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { lean_object* x_12; -x_12 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_12 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -3897,11 +4038,11 @@ lean_dec(x_5); return x_12; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { lean_object* x_14; -x_14 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +x_14 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -3911,11 +4052,11 @@ lean_dec(x_1); return x_14; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { lean_object* x_10; -x_10 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_10 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__7(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -3924,20 +4065,7 @@ lean_dec(x_1); return x_10; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -lean_object* x_7; -x_7 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__7(x_1, x_2, x_3, x_4, x_5, x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_7; -} -} -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { size_t x_11; size_t x_12; lean_object* x_13; @@ -3945,51 +4073,51 @@ x_11 = lean_unbox_usize(x_5); lean_dec(x_5); x_12 = lean_unbox_usize(x_6); lean_dec(x_6); -x_13 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12(x_1, x_2, x_3, x_4, x_11, x_12, x_7, x_8, x_9, x_10); +x_13 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11(x_1, x_2, x_3, x_4, x_11, x_12, x_7, x_8, x_9, x_10); lean_dec(x_4); return x_13; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13(x_1, x_2); +x_3 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12(x_1, x_2); lean_dec(x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; -x_7 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_5); lean_dec(x_2); return x_7; } } -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___lambda__1(x_1, x_2); +x_3 = l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___lambda__1(x_1, x_2); lean_dec(x_2); lean_dec(x_1); x_4 = lean_box(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15(x_1, x_2, x_3); +x_4 = l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14(x_1, x_2, x_3); lean_dec(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { size_t x_8; size_t x_9; lean_object* x_10; @@ -3997,13 +4125,13 @@ x_8 = lean_unbox_usize(x_2); lean_dec(x_2); x_9 = lean_unbox_usize(x_3); lean_dec(x_3); -x_10 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16(x_1, x_8, x_9, x_4, x_5, x_6, x_7); +x_10 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15(x_1, x_8, x_9, x_4, x_5, x_6, x_7); lean_dec(x_6); lean_dec(x_1); return x_10; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__17___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { size_t x_5; size_t x_6; lean_object* x_7; @@ -4011,7 +4139,7 @@ x_5 = lean_unbox_usize(x_2); lean_dec(x_2); x_6 = lean_unbox_usize(x_3); lean_dec(x_3); -x_7 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__17(x_1, x_5, x_6, x_4); +x_7 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16(x_1, x_5, x_6, x_4); lean_dec(x_1); return x_7; } @@ -4072,60 +4200,60 @@ lean_mark_persistent(l_Lean_Linter_linter_constructorNameAsVariable); lean_dec_ref(res); }l_List_forIn_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__6___lambda__1___closed__1 = _init_l_List_forIn_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__6___lambda__1___closed__1(); lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__6___lambda__1___closed__1); -l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__10___closed__1 = _init_l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__10___closed__1(); -lean_mark_persistent(l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__10___closed__1); -l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__1 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__1(); -lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__1); -l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__2 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__2(); -lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__2); -l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__3 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__3(); -lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__3); -l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__4 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__4(); -lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__4); -l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__4___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__4___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__4___closed__1); -l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___closed__1); -l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__1 = _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__1(); -lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__1); -l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__2 = _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__2(); -lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__2); -l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__3 = _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__3(); -lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__3); -l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__4 = _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__4(); -lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__4); -l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__5 = _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__5(); -lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__5); -l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__6 = _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__6(); -lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__6); -l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__7 = _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__7(); -lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__7); -l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__1 = _init_l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__1(); -lean_mark_persistent(l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__1); -l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__1); -l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__2 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__2(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__2); -l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__3 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__3(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__3); -l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__4 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__4(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__4); -l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__5 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__5(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__5); -l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__6 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__6(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__6); -l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__7 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__7(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__7); -l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__8 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__8(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__8); -l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__9 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__9(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__9); -l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__10 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__10(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__10); -l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__11 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__11(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__11); -l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__12 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__12(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__12); +l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__1 = _init_l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__1(); +lean_mark_persistent(l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__1); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__1 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__1(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__1); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__2 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__2(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__2); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__3 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__3(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__3); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__4 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__4(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__4); +l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__5___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__5___closed__1(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__5___closed__1); +l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___closed__1(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___closed__1); +l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__1 = _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__1(); +lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__1); +l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__2 = _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__2(); +lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__2); +l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__3 = _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__3(); +lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__3); +l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__4 = _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__4(); +lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__4); +l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__5 = _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__5(); +lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__5); +l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__6 = _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__6(); +lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__6); +l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__7 = _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__7(); +lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__7); +l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__1 = _init_l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__1(); +lean_mark_persistent(l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__1); +l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__1(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__1); +l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__2 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__2(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__2); +l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__3 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__3(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__3); +l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__4 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__4(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__4); +l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__5 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__5(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__5); +l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__6 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__6(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__6); +l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__7 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__7(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__7); +l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__8 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__8(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__8); +l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__9 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__9(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__9); +l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__10 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__10(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__10); +l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__11 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__11(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__11); +l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__12 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__12(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__12); l_Lean_Linter_constructorNameAsVariable___elambda__1___closed__1 = _init_l_Lean_Linter_constructorNameAsVariable___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Linter_constructorNameAsVariable___elambda__1___closed__1); l_Lean_Linter_constructorNameAsVariable___elambda__1___closed__2 = _init_l_Lean_Linter_constructorNameAsVariable___elambda__1___closed__2(); diff --git a/stage0/stdlib/Lean/Linter/UnusedVariables.c b/stage0/stdlib/Lean/Linter/UnusedVariables.c index cb150692a468..5666c1ef7969 100644 --- a/stage0/stdlib/Lean/Linter/UnusedVariables.c +++ b/stage0/stdlib/Lean/Linter/UnusedVariables.c @@ -13,652 +13,712 @@ #ifdef __cplusplus extern "C" { #endif -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__6; +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__20___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__31(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___boxed(lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316_(lean_object*); +static lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__3; LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_visitAssignments(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_UnusedVariables_collectReferences_skipDeclIdIfPresent___closed__1; -LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__2(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__3; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__6; +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__32(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_followAliases(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__5; -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__9; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4___closed__2; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_collectReferences___spec__1(lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__2; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__10; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____closed__1; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__9; +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__24___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3___closed__1; LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_insertObjImpl___rarg___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__8; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__17(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_insertObjImpl___spec__2(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__22; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__6; lean_object* lean_mk_empty_array_with_capacity(lean_object*); -static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__2; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__8; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231_(lean_object*); +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14(lean_object*, size_t, size_t); +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__11___boxed(lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__2; +static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__1; uint8_t l_Lean_Syntax_matchesIdent(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__3; -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____closed__1; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__10; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__11___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__11; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4___closed__1; -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___lambda__1(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__9; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__2; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__6; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__7; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__2; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690_(lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__8; LEAN_EXPORT lean_object* l_Lean_Linter_getUnusedVariablesIgnoreFns(lean_object*); +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PersistentArray_toArray___rarg(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__2; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107_(lean_object*); -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___lambda__1___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__9; LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_collectReferences___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987_(lean_object*); lean_object* l_Lean_ConstantInfo_type(lean_object*); -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____closed__1; LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_visitAssignments_visitEntry___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__1; +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4(lean_object*, lean_object*); lean_object* l_Lean_Syntax_getHeadInfo(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__9; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__10; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__6(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__2(lean_object*, uint8_t, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__3; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____closed__1; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__1; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__6; uint64_t l___private_Lean_Syntax_0__String_hashRange____x40_Lean_Syntax___hyg_169_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__5___boxed(lean_object**); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__4; LEAN_EXPORT lean_object* l_Lean_Linter_getUnusedVariablesIgnoreFns___boxed(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__11; -LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__8; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_collectReferences___spec__1___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_ForEachExpr_visit___spec__2(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Linter_UnusedVariables_insertObjImpl___spec__3(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__8; LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__1; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__4; size_t lean_uint64_to_usize(uint64_t); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_visitAssignments_visitNode(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__3; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___closed__2; LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_insertObjImpl___spec__1(size_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_initFn____x40_Lean_Linter_UnusedVariables___hyg_5794_(lean_object*); -LEAN_EXPORT uint8_t l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1(lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__2; +LEAN_EXPORT lean_object* l_Array_sequenceMap_loop___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_toString(lean_object*, uint8_t, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__18; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__3; +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__5; lean_object* l_Lean_Syntax_getId(lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__19; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__1; uint8_t l___private_Lean_Syntax_0__String_beqRange____x40_Lean_Syntax___hyg_95_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_getLinterUnusedVariables___boxed(lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__4; +LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_collectReferences_go___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__3(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__12; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___closed__1; lean_object* l_Array_qpartition___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__2; -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__21; -static lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___closed__1; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__2(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__16; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__8; lean_object* lean_mk_array(lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___closed__1; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__3; +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__13; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__2; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__7___closed__1; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getArgs(lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__23(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__2___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__11; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__13; uint8_t l_String_Range_includes(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__1; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__12; -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__17___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getPos_x3f(lean_object*, uint8_t); lean_object* lean_array_fget(lean_object*, lean_object*); lean_object* l_Lean_Elab_InfoTree_hasSorry(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__3; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__6(lean_object*, lean_object*, lean_object*); lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__10; static lean_object* l_Lean_Linter_UnusedVariables_unusedVariables___closed__3; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__7(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__23___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_visitAssignments_visitExpr___lambda__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_UnusedVariables_visitAssignments___closed__2; -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__4; -LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__4; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__2; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__5; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__10; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__18(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__23___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_getLinterUnusedVariablesFunArgs___boxed(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__19; +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__1; lean_object* lean_environment_find(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__3; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___closed__1; lean_object* l_Lean_Attribute_Builtin_ensureNoArgs(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__4; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_logAt___at_Lean_Elab_Command_runLinters___spec__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__22; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__30___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3___closed__2; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__3; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___closed__3; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__7; uint8_t l_Lean_Linter_getLinterValue(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__8; +static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__3; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__9; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__3; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__3___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Nat_nextPowerOfTwo_go(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__1; +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__24(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t); lean_object* l_Lean_stringToMessageData(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__1(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences___spec__16___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__18___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_EStateM_instMonad(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_insertObjImpl(lean_object*); lean_object* l_Lean_PersistentArray_toList___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__3___boxed(lean_object**); uint8_t l_List_any___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1(lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); lean_object* l_List_head_x21___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_visitAssignments_visitNode___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__4; -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__12(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__8(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__17; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__4(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_getUnusedVariablesIgnoreFns___rarg___closed__1; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Linter_getLinterUnusedVariablesFunArgs(lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__5___closed__1; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__5___closed__1; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__6; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_insertObjImpl___spec__1___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__7; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__3; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__2; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4___closed__2; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__18(lean_object*, lean_object*); lean_object* lean_string_utf8_byte_size(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__10; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__12(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__5; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____closed__1; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__4; -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__24___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__3; +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__18___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__2; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__12(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Linter_mkIgnoreFnImpl___lambda__1(lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_collectReferences___spec__5(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__3___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__8; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___boxed(lean_object**); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__3; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__8; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__13; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__2; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____closed__1; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__2; -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__2; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__11; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__1(lean_object*); static lean_object* l_Lean_Linter_mkIgnoreFnImpl___closed__2; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__2; size_t lean_ptr_addr(lean_object*); lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__5; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__2; +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__7; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__4; +LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__7(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ForEachExpr_visit___at_Lean_Linter_UnusedVariables_visitAssignments_visitExpr___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT uint8_t l_Lean_Linter_getLinterUnusedVariablesPatternVars(lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_47____closed__2; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__6; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__7; -static lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__3; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__7; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__7; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__9; +LEAN_EXPORT uint8_t l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__6; +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__4; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__18; +static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__4; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__5; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__10; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_visitAssignments_visitNode___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_sequenceMap_loop___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__6; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariablesIgnoreFnsExt; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__4; static lean_object* l_Lean_Linter_UnusedVariables_unusedVariables___closed__2; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__5___closed__1; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__5; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__3; lean_object* lean_local_ctx_find(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__8(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__13(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__7; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__29___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__1; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__13(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__5; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__8; lean_object* lean_st_ref_take(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__24; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__11; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_ForEachExpr_visit___spec__3(lean_object*); static lean_object* l_Lean_Linter_UnusedVariables_collectReferences_skipDeclIdIfPresent___closed__2; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3(lean_object*, size_t, size_t); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__6; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__3; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3___closed__1; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_86_(lean_object*); lean_object* l_Lean_declareBuiltin(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Array_sequenceMap_loop___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6___closed__2; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_insertObjImpl___spec__4(lean_object*, lean_object*, lean_object*); lean_object* l_List_filterMapTR_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__3; lean_object* l_Lean_registerPersistentEnvExtensionUnsafe___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_visitAssignments_visitExpr(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1(lean_object*, lean_object*, lean_object*); uint64_t lean_uint64_shift_right(uint64_t, uint64_t); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6___closed__2; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__11; +static lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__4; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint64_t lean_usize_to_uint64(size_t); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__2; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__14; +static lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__6; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__4___boxed(lean_object**); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__5___closed__1; lean_object* lean_nat_div(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___closed__1; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__12; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379_(lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__7; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__7; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Info_updateContext_x3f(lean_object*, lean_object*); -static lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__1; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__2___boxed(lean_object*, lean_object*, lean_object*); uint64_t l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(lean_object*); lean_object* l_Lean_PersistentEnvExtension_addEntry___rarg(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__6; uint8_t l_Lean_Syntax_Stack_matches(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__8; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_47____closed__3; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__7; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__2___closed__1; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__9; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__1___boxed(lean_object*, lean_object*); +static lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__1; LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PersistentEnvExtension_getState___rarg(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__7; lean_object* lean_eval_const(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_340____closed__1; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__8; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3___closed__2; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__15___boxed(lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t); +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_linter_unusedVariables_patternVars; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_86____closed__2; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__8(lean_object*); -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__2; lean_object* l_Lean_Elab_PartialContextInfo_mergeIntoOuter_x3f(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__20; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__2; LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__6; -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__5; -LEAN_EXPORT lean_object* l_Array_sequenceMap___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___lambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___lambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__2; lean_object* l_Lean_MessageData_ofFormat(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences___spec__16(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3___closed__2; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__1; lean_object* l_Lean_setEnv___at_Lean_registerParametricAttribute___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__1; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__4; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555_(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__2; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6___closed__1; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__24; +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_collectReferences_go(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__13; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_collectReferences_skipDeclIdIfPresent(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____closed__1; -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__8; lean_object* l_Lean_throwError___at_Lean_registerTagAttribute___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_filterMapTR_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__2(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__13; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948_(lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__4(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__3(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__11; lean_object* lean_st_mk_ref(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____closed__1; static lean_object* l_Lean_Linter_UnusedVariables_visitAssignments___closed__1; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__7(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); static lean_object* l_Lean_Linter_UnusedVariables_unusedVariables___closed__1; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__6; -LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__4; uint8_t l_Lean_MessageData_hasTag(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_unusedVariables; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__1; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601_(lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125_(lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__8; LEAN_EXPORT lean_object* l_Lean_Linter_mkIgnoreFnImpl___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__1; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__3; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_visitAssignments___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19(lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__7; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1(lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__3; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__11(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); static lean_object* l_Lean_Linter_mkIgnoreFnImpl___closed__5; -static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__5; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__3; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__7; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__2; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__2; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__4; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__10; -static lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__2; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__5; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__1; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__2; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__9; +static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__6; +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__32___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__6; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__1; uint64_t l_Lean_Expr_hash(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__3; -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__20(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__3; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__9; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__6; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__4; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__5; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__8; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__6; +LEAN_EXPORT lean_object* l_Array_sequenceMap___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__1___boxed(lean_object*, lean_object*); lean_object* l_List_lengthTRAux___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__4(lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_mkIgnoreFnImpl___closed__3; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__13; -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Elab_Command_instMonadCommandElabM; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__1; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__4; +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___closed__1; uint8_t lean_name_eq(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__5; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__18(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6(lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__8; +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__23(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__1(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_MessageData_isUnusedVariableWarning___lambda__1(lean_object*); -LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_visitAssignments___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__4; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__1; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__2___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__1; -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_collectReferences___spec__14(lean_object*, lean_object*); -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__16; +static lean_object* l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__1; +uint8_t l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__7; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__4___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__3; lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_addBuiltinUnusedVariablesIgnoreFn(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__8; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__3; static lean_object* l_Lean_Linter_mkIgnoreFnImpl___closed__4; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__1; lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__16(lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__21; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__1; uint8_t l_Lean_Syntax_matchesNull(lean_object*, lean_object*); static lean_object* l_Lean_Linter_addBuiltinUnusedVariablesIgnoreFn___closed__1; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__4; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__7(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__20___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); static lean_object* l_Lean_Linter_mkIgnoreFnImpl___closed__1; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__15; LEAN_EXPORT lean_object* l_Lean_Linter_builtinUnusedVariablesIgnoreFnsRef; -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__2; -LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__7(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__1; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379____closed__1; uint8_t l_Lean_Syntax_isIdent(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__3; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__6; -static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__1; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__5; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__1; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__12; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_visitAssignments_visitExpr___lambda__1(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__3(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__9; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__3; -LEAN_EXPORT uint8_t l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__1(lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__7___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__2; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__1; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__5(lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__3___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__11; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__3; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__7; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__20; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__7; +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__2; static lean_object* l_Lean_Linter_getLinterUnusedVariables___closed__1; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__2; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__9; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__11; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__3(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_sequenceMap___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_visitAssignments_visitNode___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_linter_unusedVariables_analyzeTactics; lean_object* l_Lean_Elab_Command_addLinter(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16___lambda__1___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__3___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__2; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__17(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_ForEachExpr_visit___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_insertObjImpl___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____closed__1; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__15; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__5; +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___lambda__1___boxed(lean_object*, lean_object*); lean_object* l_Lean_Option_register___at_Lean_Elab_initFn____x40_Lean_Elab_AutoBound___hyg_6____spec__1(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__1; -static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__1; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__3; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__7; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3___closed__1; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__1; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__4; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475_(lean_object*); +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); +static lean_object* l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__2; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__3; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__4; LEAN_EXPORT uint8_t l_Lean_MessageData_isUnusedVariableWarning(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_visitAssignments_visitNode___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__6; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, uint8_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_userName(lean_object*); lean_object* l_Substring_nextn(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277_(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__4; -static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__3; -static lean_object* l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__3; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____closed__1; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__5; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__1; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__2; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__1; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6___closed__1; lean_object* l_panic___at_Lean_Parser_ParserState_mkUnexpectedTokenErrors___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__23___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__7; LEAN_EXPORT lean_object* l_IO_ofExcept___at_Lean_Linter_mkIgnoreFnImpl___spec__1(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__10; +static lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__7; +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_followAliases___boxed(lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__2; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__4(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__9; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static size_t l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__3___closed__1; LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_visitAssignments___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____closed__1; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_sequenceMap_loop___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__1; uint8_t l_Lean_Name_hasMacroScopes(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__4; -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__2(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____closed__1; static lean_object* l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___lambda__2___closed__1; lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_ForEachExpr_visit___spec__6(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_linter_unusedVariables; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____closed__1; uint8_t l_String_Range_contains(lean_object*, lean_object*, uint8_t); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__4___boxed(lean_object**); -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__8; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__15(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__20(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__5; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__5; lean_object* l_Lean_Expr_app___override(lean_object*, lean_object*); static lean_object* l_Lean_Linter_mkIgnoreFnImpl___closed__6; lean_object* lean_string_length(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__4; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__5(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__20___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_collectReferences(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____closed__1; uint8_t l_Lean_Syntax_hasArgs(lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Linter_getLinterUnusedVariables(lean_object*); -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__2; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__5; -static lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640_(lean_object*); +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_findStack_x3f(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_MessageData_isUnusedVariableWarning___lambda__1___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_getUnusedVariablesIgnoreFns___rarg___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__1; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__1; uint8_t lean_nat_dec_lt(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982_(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__3; static lean_object* l_Lean_MessageData_isUnusedVariableWarning___closed__1; -LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____closed__1; +LEAN_EXPORT uint8_t l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__1(lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__9; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__9(lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_PersistentHashMap_insert___at_Lean_MVarId_assign___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_visitAssignments_visitExpr___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_isOfKind___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_getUnusedVariablesIgnoreFns___rarg(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__3; +static lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__2; lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__1___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__2___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__3; +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____closed__1; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_getConstInfo___at_Lean_registerInitAttrUnsafe___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__8; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__12; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__4(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__4; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____closed__1; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__8(lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_initFn____x40_Lean_Linter_UnusedVariables___hyg_6304_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__6___boxed(lean_object**); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021_(lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__2; +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14___lambda__1(lean_object*); uint8_t l_Lean_Expr_isConstOf(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__8; +LEAN_EXPORT uint8_t l_Lean_PersistentArray_anyMAux___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__12(lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__9; LEAN_EXPORT lean_object* l_Lean_MessageData_isUnusedVariableWarning___boxed(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__6; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__10; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__5; LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__7; uint64_t lean_uint64_xor(uint64_t, uint64_t); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__1; -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__23(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t); uint8_t l_Lean_Syntax_isNone(lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* lean_panic_fn(lean_object*, lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_86____closed__4; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__2___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_visitAssignments_visitNode___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__11(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703_(lean_object*); -static lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__4; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192_(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__9; +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14___lambda__1___boxed(lean_object*); +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____closed__1; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4___closed__1; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__2(lean_object*, lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387_(lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__29(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__2(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__7; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__14; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____closed__1; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6(lean_object*); lean_object* lean_nat_mul(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__5; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__10; +static lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__2; lean_object* l_Lean_Syntax_getRange_x3f(lean_object*, uint8_t); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); +static lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Linter_mkIgnoreFnImpl___lambda__1___boxed(lean_object*); lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3___closed__2; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__12; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__13___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__2; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__4; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__4; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Info_range_x3f(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__3(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__3; +static lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__5; +lean_object* l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_registerBuiltinAttribute(lean_object*, lean_object*); +static lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14___closed__1; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__10; lean_object* l_List_reverse___rarg(lean_object*); -static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__3; -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__24(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3(lean_object*, size_t, size_t); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__12; uint8_t l___private_Lean_Attributes_0__Lean_beqAttributeKind____x40_Lean_Attributes___hyg_162_(uint8_t, uint8_t); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__9; -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__4; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__12; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_86____closed__1; size_t lean_usize_sub(size_t, size_t); +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Elab_Command_instInhabitedScope; lean_object* lean_array_mk(lean_object*); +LEAN_EXPORT lean_object* l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22(lean_object*, uint8_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__5(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443_(lean_object*); static lean_object* l_panic___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__8___closed__1; -static lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___lambda__2___closed__1; -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__17(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__17; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__4; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_instantiateMVarsCore(lean_object*, lean_object*); uint8_t l_Substring_beq(lean_object*, lean_object*); -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__5; size_t lean_usize_add(size_t, size_t); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__14(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__2; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__13(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_hasFVar(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__3; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016_(lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_collectReferences___spec__10(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__4; +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_KVMap_findCore(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__4; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__9(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__2; lean_object* lean_array_uget(lean_object*, size_t); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__14; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__9(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); size_t lean_array_size(lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_47_(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__7; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__3; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__3; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__6; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8_(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__15(lean_object*, lean_object*); lean_object* lean_io_error_to_string(lean_object*); lean_object* l_instInhabitedOfMonad___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_insertObjImpl___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__14; lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6___boxed(lean_object*); -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__2(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__2___boxed(lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Elab_InfoTree_findInfo_x3f(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__6; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__6; +static lean_object* l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__4; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__12; LEAN_EXPORT lean_object* l_Lean_Linter_getLinterUnusedVariablesPatternVars___boxed(lean_object*); lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__6; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_47____closed__5; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__2; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__6; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3___closed__1; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__9; +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1(lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__5; +static lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___closed__1; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_47____closed__1; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_UnusedVariables_visitAssignments___closed__3; -LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__11(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__11; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ForEachExpr_visit___at_Lean_Linter_UnusedVariables_visitAssignments_visitExpr___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_mkIgnoreFnImpl___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____closed__1; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__5; lean_object* lean_string_append(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_insertObjImpl___spec__4___at_Lean_Linter_UnusedVariables_insertObjImpl___spec__5(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_followAliases___spec__1___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__11; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__10(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_mkIgnoreFnImpl___closed__7; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__11; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1(lean_object*, lean_object*, lean_object*); lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Syntax_SepArray_getElems___spec__1(lean_object*, size_t, size_t, lean_object*); lean_object* lean_array_get_size(lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__7___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__2(lean_object*, lean_object*); uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__8; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_47____closed__4; LEAN_EXPORT lean_object* l_Lean_Linter_mkIgnoreFnImpl(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__7; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__5; +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__13(lean_object*, size_t, size_t); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__1; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__3; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__7; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742_(lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); -static lean_object* l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__2; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__11___boxed(lean_object*, lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__5; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__3; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__23; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__30(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_followAliases___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_86____closed__5; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__2; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__9; lean_object* lean_nat_add(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__2; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__4; lean_object* l_Lean_Elab_Info_stx(lean_object*); lean_object* l_EStateM_bind___rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_340_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__3; -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__4; +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_visitAssignments_visitEntry(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__6; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__6___boxed(lean_object**); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__5___boxed(lean_object**); -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__17___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_sequenceMap___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__1___boxed(lean_object*, lean_object*); -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16___lambda__1(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__3; +LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__12___boxed(lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__3; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t); -static lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__2; -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__5; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_throwError___at_Lean_Attribute_Builtin_ensureNoArgs___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__6; -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651_(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__23; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__31___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__19(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__4; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__1; LEAN_EXPORT lean_object* l_Lean_Linter_linter_unusedVariables_funArgs; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_UnusedVariables_collectReferences___spec__17(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Lean_PersistentArray_anyM___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__11(lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__10; lean_object* l_Lean_MessageData_ofName(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__2; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__1; lean_object* l___private_Init_Data_Repr_0__Nat_reprFast(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__5; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__4; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__4; +static lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_insertObjImpl___rarg(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__10; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__12; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__7; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__4; +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__2(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__14(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__2___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_86____closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences___spec__16___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__5; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__3; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__1___boxed(lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____closed__1; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__3(lean_object*); lean_object* l_List_get_x3f___rarg(lean_object*, lean_object*); lean_object* l_ReaderT_instMonad___rarg(lean_object*); size_t lean_usize_land(size_t, size_t); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__5; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__9; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__5; LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__9; -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__3; uint8_t l_Lean_Elab_Info_contains(lean_object*, lean_object*, uint8_t); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___boxed(lean_object**); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____closed__1; uint8_t l_Lean_MessageLog_hasErrors(lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__5; static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__1() { _start: { @@ -887,6 +947,72 @@ x_5 = l_Lean_Option_register___at_Lean_Elab_initFn____x40_Lean_Elab_AutoBound___ return x_5; } } +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("analyzeTactics", 14, 14); +return x_1; +} +} +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__2; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__1; +x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("enable analysis of local variables in presence of tactic proofs\n\nBy default, the linter will limit itself to linting a declaration's parameters whenever tactic proofs are present as these can be expensive to analyze. Enabling this option extends linting to local variables both inside and outside tactic proofs, though it can also lead to some false negatives as intermediate tactic states may reference some variables without the declaration ultimately depending on them.", 472, 472); +return x_1; +} +} +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__4() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = 0; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__3; +x_4 = lean_box(x_1); +x_5 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_5, 0, x_4); +lean_ctor_set(x_5, 1, x_2); +lean_ctor_set(x_5, 2, x_3); +return x_5; +} +} +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__8; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__1; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__2; +x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__1; +x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__2; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__4; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__5; +x_5 = l_Lean_Option_register___at_Lean_Elab_initFn____x40_Lean_Elab_AutoBound___hyg_6____spec__1(x_2, x_3, x_4, x_1); +return x_5; +} +} static lean_object* _init_l_Lean_Linter_getLinterUnusedVariables___closed__1() { _start: { @@ -1340,7 +1466,7 @@ lean_dec(x_1); return x_7; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_340____closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379____closed__1() { _start: { lean_object* x_1; lean_object* x_2; @@ -1349,11 +1475,11 @@ x_2 = lean_array_mk(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_340_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; uint8_t x_4; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_340____closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379____closed__1; x_3 = lean_st_mk_ref(x_2, x_1); x_4 = !lean_is_exclusive(x_3); if (x_4 == 0) @@ -1416,7 +1542,7 @@ return x_12; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____spec__1(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____spec__1(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { uint8_t x_7; @@ -1479,7 +1605,7 @@ return x_20; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____spec__2(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____spec__2(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { uint8_t x_7; @@ -1522,7 +1648,7 @@ x_19 = 0; x_20 = lean_usize_of_nat(x_9); lean_dec(x_9); lean_inc(x_5); -x_21 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____spec__1(x_8, x_19, x_20, x_4, x_5, x_6); +x_21 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____spec__1(x_8, x_19, x_20, x_4, x_5, x_6); lean_dec(x_8); if (lean_obj_tag(x_21) == 0) { @@ -1576,7 +1702,7 @@ return x_31; } } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__1(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; uint8_t x_4; @@ -1602,7 +1728,7 @@ return x_7; } } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__2(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__2(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; lean_object* x_4; lean_object* x_5; @@ -1616,7 +1742,7 @@ lean_ctor_set(x_5, 1, x_2); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_5; uint8_t x_6; @@ -1666,7 +1792,7 @@ lean_free_object(x_5); x_17 = 0; x_18 = lean_usize_of_nat(x_9); lean_dec(x_9); -x_19 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____spec__2(x_1, x_17, x_18, x_7, x_2, x_8); +x_19 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____spec__2(x_1, x_17, x_18, x_7, x_2, x_8); if (lean_obj_tag(x_19) == 0) { uint8_t x_20; @@ -1774,7 +1900,7 @@ size_t x_45; size_t x_46; lean_object* x_47; x_45 = 0; x_46 = lean_usize_of_nat(x_35); lean_dec(x_35); -x_47 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____spec__2(x_1, x_45, x_46, x_33, x_2, x_34); +x_47 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____spec__2(x_1, x_45, x_46, x_33, x_2, x_34); if (lean_obj_tag(x_47) == 0) { lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; @@ -1832,7 +1958,7 @@ return x_57; } } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__4(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__4(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; @@ -1911,7 +2037,7 @@ return x_23; } } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__5(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__5(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; @@ -1923,7 +2049,7 @@ x_4 = lean_array_mk(x_3); return x_4; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6___closed__1() { _start: { lean_object* x_1; @@ -1931,17 +2057,17 @@ x_1 = lean_mk_string_unchecked("number of local entries: ", 25, 25); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6___closed__1; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6___closed__1; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; @@ -1951,14 +2077,14 @@ x_4 = l_List_lengthTRAux___rarg(x_2, x_3); x_5 = l___private_Init_Data_Repr_0__Nat_reprFast(x_4); x_6 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_6, 0, x_5); -x_7 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6___closed__2; +x_7 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6___closed__2; x_8 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_8, 0, x_7); lean_ctor_set(x_8, 1, x_6); return x_8; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__1() { _start: { lean_object* x_1; @@ -1966,87 +2092,87 @@ x_1 = lean_mk_string_unchecked("unusedVariablesIgnoreFnsExt", 27, 27); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__8; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__1; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__1; x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__3() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__3() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__1), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__1), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__4() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__4() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__2), 2, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__2), 2, 0); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__5() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__4; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__4; x_3 = lean_alloc_closure((void*)(l_EStateM_bind___rarg), 3, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__6() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__6() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__3___boxed), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__3___boxed), 3, 0); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__7() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__7() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__4), 2, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__4), 2, 0); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__8() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__8() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__5), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__5), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__9() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__9() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6___boxed), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6___boxed), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__10() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__2; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__5; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__6; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__7; -x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__8; -x_6 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__9; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__2; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__5; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__6; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__7; +x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__8; +x_6 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__9; x_7 = lean_alloc_ctor(0, 6, 0); lean_ctor_set(x_7, 0, x_1); lean_ctor_set(x_7, 1, x_2); @@ -2057,16 +2183,16 @@ lean_ctor_set(x_7, 5, x_6); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__10; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__10; x_3 = l_Lean_registerPersistentEnvExtensionUnsafe___rarg(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { size_t x_7; size_t x_8; lean_object* x_9; @@ -2074,12 +2200,12 @@ x_7 = lean_unbox_usize(x_2); lean_dec(x_2); x_8 = lean_unbox_usize(x_3); lean_dec(x_3); -x_9 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____spec__1(x_1, x_7, x_8, x_4, x_5, x_6); +x_9 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____spec__1(x_1, x_7, x_8, x_4, x_5, x_6); lean_dec(x_1); return x_9; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { size_t x_7; size_t x_8; lean_object* x_9; @@ -2087,30 +2213,30 @@ x_7 = lean_unbox_usize(x_2); lean_dec(x_2); x_8 = lean_unbox_usize(x_3); lean_dec(x_3); -x_9 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____spec__2(x_1, x_7, x_8, x_4, x_5, x_6); +x_9 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____spec__2(x_1, x_7, x_8, x_4, x_5, x_6); lean_dec(x_1); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__3(x_1, x_2, x_3); +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__3(x_1, x_2, x_3); lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6___boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6___boxed(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6(x_1); +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6(x_1); lean_dec(x_1); return x_2; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___closed__1() { _start: { lean_object* x_1; @@ -2118,28 +2244,28 @@ x_1 = lean_mk_string_unchecked("addBuiltinUnusedVariablesIgnoreFn", 33, 33); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__8; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__1; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___closed__1; x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__3() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__2; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___closed__2; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; @@ -2150,13 +2276,13 @@ lean_dec(x_6); x_8 = lean_box(0); lean_inc(x_1); x_9 = l_Lean_Expr_const___override(x_1, x_8); -x_10 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__3; +x_10 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___closed__3; x_11 = l_Lean_Expr_app___override(x_10, x_9); x_12 = l_Lean_declareBuiltin(x_1, x_11, x_3, x_4, x_7); return x_12; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__1() { _start: { lean_object* x_1; @@ -2164,16 +2290,16 @@ x_1 = lean_mk_string_unchecked("invalid attribute '", 19, 19); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__1; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__3() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__3() { _start: { lean_object* x_1; lean_object* x_2; @@ -2182,7 +2308,7 @@ x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; @@ -2206,11 +2332,11 @@ if (x_12 == 0) lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_dec(x_1); x_13 = l_Lean_MessageData_ofName(x_2); -x_14 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__2; +x_14 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__2; x_15 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_15, 0, x_14); lean_ctor_set(x_15, 1, x_13); -x_16 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__3; +x_16 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__3; x_17 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_17, 0, x_15); lean_ctor_set(x_17, 1, x_16); @@ -2239,7 +2365,7 @@ else lean_object* x_23; lean_object* x_24; lean_dec(x_2); x_23 = lean_box(0); -x_24 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1(x_1, x_23, x_4, x_5, x_9); +x_24 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1(x_1, x_23, x_4, x_5, x_9); return x_24; } } @@ -2269,7 +2395,7 @@ return x_28; } } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3___closed__1() { _start: { lean_object* x_1; @@ -2277,16 +2403,16 @@ x_1 = lean_mk_string_unchecked("', must be global", 17, 17); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3___closed__1; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; @@ -2305,11 +2431,11 @@ if (x_11 == 0) lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_dec(x_2); x_12 = l_Lean_MessageData_ofName(x_1); -x_13 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__2; +x_13 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__2; x_14 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_14, 0, x_13); lean_ctor_set(x_14, 1, x_12); -x_15 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3___closed__2; +x_15 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3___closed__2; x_16 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_16, 0, x_14); lean_ctor_set(x_16, 1, x_15); @@ -2338,7 +2464,7 @@ else { lean_object* x_22; lean_object* x_23; x_22 = lean_box(0); -x_23 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2(x_2, x_1, x_22, x_5, x_6, x_9); +x_23 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2(x_2, x_1, x_22, x_5, x_6, x_9); lean_dec(x_5); return x_23; } @@ -2370,7 +2496,7 @@ return x_27; } } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4___closed__1() { _start: { lean_object* x_1; @@ -2378,25 +2504,25 @@ x_1 = lean_mk_string_unchecked("attribute cannot be erased", 26, 26); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4___closed__1; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; -x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4___closed__2; +x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4___closed__2; x_6 = l_Lean_throwError___at_Lean_Attribute_Builtin_ensureNoArgs___spec__2(x_5, x_2, x_3, x_4); return x_6; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__5___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__5___closed__1() { _start: { lean_object* x_1; @@ -2404,7 +2530,7 @@ x_1 = l_Lean_Linter_unusedVariablesIgnoreFnsExt; return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; uint8_t x_7; @@ -2445,7 +2571,7 @@ lean_inc(x_20); lean_dec(x_18); lean_ctor_set(x_6, 1, x_19); lean_ctor_set(x_6, 0, x_1); -x_21 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__5___closed__1; +x_21 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__5___closed__1; x_22 = l_Lean_PersistentEnvExtension_addEntry___rarg(x_21, x_10, x_6); x_23 = l_Lean_setEnv___at_Lean_registerParametricAttribute___spec__3(x_22, x_3, x_4, x_20); return x_23; @@ -2521,7 +2647,7 @@ lean_inc(x_43); lean_dec(x_41); lean_ctor_set(x_6, 1, x_42); lean_ctor_set(x_6, 0, x_1); -x_44 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__5___closed__1; +x_44 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__5___closed__1; x_45 = l_Lean_PersistentEnvExtension_addEntry___rarg(x_44, x_10, x_6); x_46 = l_Lean_setEnv___at_Lean_registerParametricAttribute___spec__3(x_45, x_3, x_4, x_43); return x_46; @@ -2611,7 +2737,7 @@ lean_dec(x_65); x_68 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_68, 0, x_1); lean_ctor_set(x_68, 1, x_66); -x_69 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__5___closed__1; +x_69 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__5___closed__1; x_70 = l_Lean_PersistentEnvExtension_addEntry___rarg(x_69, x_56, x_68); x_71 = l_Lean_setEnv___at_Lean_registerParametricAttribute___spec__3(x_70, x_3, x_4, x_67); return x_71; @@ -2653,7 +2779,7 @@ return x_79; } } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; @@ -2677,11 +2803,11 @@ if (x_12 == 0) lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_dec(x_1); x_13 = l_Lean_MessageData_ofName(x_2); -x_14 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__2; +x_14 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__2; x_15 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_15, 0, x_14); lean_ctor_set(x_15, 1, x_13); -x_16 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__3; +x_16 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__3; x_17 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_17, 0, x_15); lean_ctor_set(x_17, 1, x_16); @@ -2710,7 +2836,7 @@ else lean_object* x_23; lean_object* x_24; lean_dec(x_2); x_23 = lean_box(0); -x_24 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__5(x_1, x_23, x_4, x_5, x_9); +x_24 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__5(x_1, x_23, x_4, x_5, x_9); return x_24; } } @@ -2740,7 +2866,7 @@ return x_28; } } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; @@ -2759,11 +2885,11 @@ if (x_11 == 0) lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_dec(x_2); x_12 = l_Lean_MessageData_ofName(x_1); -x_13 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__2; +x_13 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__2; x_14 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_14, 0, x_13); lean_ctor_set(x_14, 1, x_12); -x_15 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3___closed__2; +x_15 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3___closed__2; x_16 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_16, 0, x_14); lean_ctor_set(x_16, 1, x_15); @@ -2792,7 +2918,7 @@ else { lean_object* x_22; lean_object* x_23; x_22 = lean_box(0); -x_23 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__6(x_2, x_1, x_22, x_5, x_6, x_9); +x_23 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__6(x_2, x_1, x_22, x_5, x_6, x_9); lean_dec(x_5); return x_23; } @@ -2824,7 +2950,7 @@ return x_27; } } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__1() { _start: { lean_object* x_1; @@ -2832,17 +2958,17 @@ x_1 = lean_mk_string_unchecked("builtin_unused_variables_ignore_fn", 34, 34); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__3() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -2852,17 +2978,17 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__4() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__3; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__3; x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__8; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__5() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__5() { _start: { lean_object* x_1; @@ -2870,17 +2996,17 @@ x_1 = lean_mk_string_unchecked("initFn", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__6() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__4; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__5; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__4; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__5; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__7() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__7() { _start: { lean_object* x_1; @@ -2888,37 +3014,37 @@ x_1 = lean_mk_string_unchecked("_@", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__8() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__6; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__7; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__6; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__7; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__9() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__8; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__8; x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__10() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__9; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__9; x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__8; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__11() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__11() { _start: { lean_object* x_1; @@ -2926,17 +3052,17 @@ x_1 = lean_mk_string_unchecked("UnusedVariables", 15, 15); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__12() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__10; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__11; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__10; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__11; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__13() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__13() { _start: { lean_object* x_1; @@ -2944,27 +3070,27 @@ x_1 = lean_mk_string_unchecked("_hyg", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__14() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__12; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__13; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__12; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__13; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__15() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__14; -x_2 = lean_unsigned_to_nat(601u); +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__14; +x_2 = lean_unsigned_to_nat(640u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__16() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__16() { _start: { lean_object* x_1; @@ -2972,7 +3098,7 @@ x_1 = lean_mk_string_unchecked("(builtin) ", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__17() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__17() { _start: { lean_object* x_1; @@ -2980,23 +3106,23 @@ x_1 = lean_mk_string_unchecked("Marks a function of type `Lean.Linter.IgnoreFunc return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__18() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__18() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__16; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__17; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__16; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__17; x_3 = lean_string_append(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__19() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__19() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__15; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__2; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__18; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__15; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__2; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__18; x_4 = 1; x_5 = lean_alloc_ctor(0, 3, 1); lean_ctor_set(x_5, 0, x_1); @@ -3006,15 +3132,15 @@ lean_ctor_set_uint8(x_5, sizeof(void*)*3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__20() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__20() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4___boxed), 4, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4___boxed), 4, 0); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__21() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__21() { _start: { lean_object* x_1; @@ -3022,33 +3148,33 @@ x_1 = lean_mk_string_unchecked("unused_variables_ignore_fn", 26, 26); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__22() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__22() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__21; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__21; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__23() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__23() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__4; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__17; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__17; x_3 = lean_string_append(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__24() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__24() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__15; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__22; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__23; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__15; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__22; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__23; x_4 = 1; x_5 = lean_alloc_ctor(0, 3, 1); lean_ctor_set(x_5, 0, x_1); @@ -3058,15 +3184,15 @@ lean_ctor_set_uint8(x_5, sizeof(void*)*3, x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__2; -x_3 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3___boxed), 7, 1); +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__2; +x_3 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3___boxed), 7, 1); lean_closure_set(x_3, 0, x_2); -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__19; -x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__20; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__19; +x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__20; x_6 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_6, 0, x_4); lean_ctor_set(x_6, 1, x_3); @@ -3078,10 +3204,10 @@ lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_o x_8 = lean_ctor_get(x_7, 1); lean_inc(x_8); lean_dec(x_7); -x_9 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__22; -x_10 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__7___boxed), 7, 1); +x_9 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__22; +x_10 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__7___boxed), 7, 1); lean_closure_set(x_10, 0, x_9); -x_11 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__24; +x_11 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__24; x_12 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_12, 0, x_11); lean_ctor_set(x_12, 1, x_10); @@ -3113,84 +3239,84 @@ return x_17; } } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; -x_6 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1(x_1, x_2, x_3, x_4, x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; -x_7 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { uint8_t x_8; lean_object* x_9; x_8 = lean_unbox(x_4); lean_dec(x_4); -x_9 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3(x_1, x_2, x_3, x_8, x_5, x_6, x_7); +x_9 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3(x_1, x_2, x_3, x_8, x_5, x_6, x_7); lean_dec(x_6); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4(x_1, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; -x_6 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__5(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__5(x_1, x_2, x_3, x_4, x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; -x_7 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__6(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__6(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { uint8_t x_8; lean_object* x_9; x_8 = lean_unbox(x_4); lean_dec(x_4); -x_9 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__7(x_1, x_2, x_3, x_8, x_5, x_6, x_7); +x_9 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__7(x_1, x_2, x_3, x_8, x_5, x_6, x_7); lean_dec(x_6); return x_9; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__1() { _start: { lean_object* x_1; @@ -3198,27 +3324,27 @@ x_1 = lean_mk_string_unchecked("null", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__2; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__2; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4() { _start: { lean_object* x_1; @@ -3226,7 +3352,7 @@ x_1 = lean_mk_string_unchecked("Parser", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5() { _start: { lean_object* x_1; @@ -3234,7 +3360,7 @@ x_1 = lean_mk_string_unchecked("Command", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__6() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__6() { _start: { lean_object* x_1; @@ -3242,114 +3368,114 @@ x_1 = lean_mk_string_unchecked("variable", 8, 8); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__7() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__6; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__6; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__8() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__8() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__7; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__7; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__9() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__8; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__8; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__10() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__9; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__9; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__11() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__10; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__10; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__12() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__11; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__11; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; uint8_t x_5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__12; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__12; x_5 = l_Lean_Syntax_Stack_matches(x_2, x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___boxed), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___boxed), 3, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____closed__1; x_3 = l_Lean_Linter_addBuiltinUnusedVariablesIgnoreFn(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1(x_1, x_2, x_3); +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1(x_1, x_2, x_3); lean_dec(x_3); lean_dec(x_1); x_5 = lean_box(x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__1() { _start: { lean_object* x_1; @@ -3357,114 +3483,114 @@ x_1 = lean_mk_string_unchecked("structure", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__1; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__3() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__2; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__2; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__4() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__3; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__5() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__4; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__4; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__6() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__5; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__5; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__7() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__6; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__6; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; uint8_t x_5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__7; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__7; x_5 = l_Lean_Syntax_Stack_matches(x_2, x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___boxed), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___boxed), 3, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____closed__1; x_3 = l_Lean_Linter_addBuiltinUnusedVariablesIgnoreFn(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1(x_1, x_2, x_3); +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1(x_1, x_2, x_3); lean_dec(x_3); lean_dec(x_1); x_5 = lean_box(x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__1() { _start: { lean_object* x_1; @@ -3472,89 +3598,89 @@ x_1 = lean_mk_string_unchecked("inductive", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__1; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__3() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__2; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__2; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__4() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__3; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__5() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__4; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__4; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__6() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__5; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__5; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__7() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__6; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__6; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__8() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__7; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__7; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__9() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__9() { _start: { lean_object* x_1; @@ -3562,19 +3688,19 @@ x_1 = lean_mk_string_unchecked("optDeclSig", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__10() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__9; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__9; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__11() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__11() { _start: { lean_object* x_1; @@ -3582,47 +3708,47 @@ x_1 = lean_mk_string_unchecked("declSig", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__12() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__11; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__11; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__13() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__12; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__12; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__14() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__10; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__13; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__10; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__13; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; uint8_t x_5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__8; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__8; lean_inc(x_2); x_5 = l_Lean_Syntax_Stack_matches(x_2, x_4); if (x_5 == 0) @@ -3670,7 +3796,7 @@ else lean_object* x_16; lean_object* x_17; uint8_t x_18; x_16 = lean_alloc_closure((void*)(l_Lean_Syntax_isOfKind___boxed), 2, 1); lean_closure_set(x_16, 0, x_11); -x_17 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__14; +x_17 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__14; x_18 = l_List_any___rarg(x_17, x_16); return x_18; } @@ -3678,45 +3804,45 @@ return x_18; } } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___boxed), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___boxed), 3, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____closed__1; x_3 = l_Lean_Linter_addBuiltinUnusedVariablesIgnoreFn(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1(x_1, x_2, x_3); +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1(x_1, x_2, x_3); lean_dec(x_3); lean_dec(x_1); x_5 = lean_box(x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__1() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__10; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__10; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -3728,55 +3854,55 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__3() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__1; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__2; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__2; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__4() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__3; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__3; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__5() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__4; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__4; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__6() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__5; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__5; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__7() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__7() { _start: { lean_object* x_1; @@ -3784,19 +3910,19 @@ x_1 = lean_mk_string_unchecked("ctor", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__8() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__7; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__7; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__9() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__9() { _start: { lean_object* x_1; @@ -3804,47 +3930,47 @@ x_1 = lean_mk_string_unchecked("structSimpleBinder", 18, 18); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__10() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__9; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__9; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__11() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__10; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__10; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__12() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__8; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__11; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__8; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__11; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; uint8_t x_5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__6; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__6; lean_inc(x_2); x_5 = l_Lean_Syntax_Stack_matches(x_2, x_4); if (x_5 == 0) @@ -3877,100 +4003,100 @@ lean_inc(x_11); lean_dec(x_10); x_12 = lean_alloc_closure((void*)(l_Lean_Syntax_isOfKind___boxed), 2, 1); lean_closure_set(x_12, 0, x_11); -x_13 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__12; +x_13 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__12; x_14 = l_List_any___rarg(x_13, x_12); return x_14; } } } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___boxed), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___boxed), 3, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____closed__1; x_3 = l_Lean_Linter_addBuiltinUnusedVariablesIgnoreFn(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1(x_1, x_2, x_3); +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1(x_1, x_2, x_3); lean_dec(x_3); lean_dec(x_1); x_5 = lean_box(x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__1() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__12; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__12; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__1; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__2; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__2; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__3() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__2; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__2; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__4() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__3; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__5() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__4; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__4; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__6() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__6() { _start: { lean_object* x_1; @@ -3978,19 +4104,19 @@ x_1 = lean_mk_string_unchecked("opaque", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__7() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__6; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__6; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__8() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__8() { _start: { lean_object* x_1; @@ -3998,47 +4124,47 @@ x_1 = lean_mk_string_unchecked("axiom", 5, 5); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__9() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__8; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__8; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__10() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__9; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__9; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__11() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__10; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__7; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__10; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; uint8_t x_5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__5; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__5; lean_inc(x_2); x_5 = l_Lean_Syntax_Stack_matches(x_2, x_4); if (x_5 == 0) @@ -4071,42 +4197,42 @@ lean_inc(x_11); lean_dec(x_10); x_12 = lean_alloc_closure((void*)(l_Lean_Syntax_isOfKind___boxed), 2, 1); lean_closure_set(x_12, 0, x_11); -x_13 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__11; +x_13 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__11; x_14 = l_List_any___rarg(x_13, x_12); return x_14; } } } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___boxed), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___boxed), 3, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____closed__1; x_3 = l_Lean_Linter_addBuiltinUnusedVariablesIgnoreFn(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1(x_1, x_2, x_3); +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1(x_1, x_2, x_3); lean_dec(x_3); lean_dec(x_1); x_5 = lean_box(x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Array_sequenceMap_loop___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Array_sequenceMap_loop___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; uint8_t x_7; @@ -4175,18 +4301,18 @@ return x_20; } } } -LEAN_EXPORT lean_object* l_Array_sequenceMap___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_sequenceMap___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__1(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_3 = lean_array_get_size(x_1); x_4 = lean_mk_empty_array_with_capacity(x_3); x_5 = lean_unsigned_to_nat(0u); -x_6 = l_Array_sequenceMap_loop___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__2(x_1, x_2, x_3, x_5, x_4); +x_6 = l_Array_sequenceMap_loop___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__2(x_1, x_2, x_3, x_5, x_4); return x_6; } } -static lean_object* _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__1() { +static lean_object* _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__1() { _start: { lean_object* x_1; @@ -4194,7 +4320,7 @@ x_1 = lean_mk_string_unchecked("Attr", 4, 4); return x_1; } } -static lean_object* _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__2() { +static lean_object* _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__2() { _start: { lean_object* x_1; @@ -4202,19 +4328,19 @@ x_1 = lean_mk_string_unchecked("extern", 6, 6); return x_1; } } -static lean_object* _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__3() { +static lean_object* _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__1; -x_4 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__2; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__1; +x_4 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__2; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__4() { +static lean_object* _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__4() { _start: { lean_object* x_1; @@ -4222,19 +4348,19 @@ x_1 = lean_mk_string_unchecked("simple", 6, 6); return x_1; } } -static lean_object* _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__5() { +static lean_object* _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__1; -x_4 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__4; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__1; +x_4 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__4; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__6() { +static lean_object* _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__6() { _start: { lean_object* x_1; @@ -4242,17 +4368,17 @@ x_1 = lean_mk_string_unchecked("implemented_by", 14, 14); return x_1; } } -static lean_object* _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__7() { +static lean_object* _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__6; +x_2 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3(lean_object* x_1, size_t x_2, size_t x_3) { +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3(lean_object* x_1, size_t x_2, size_t x_3) { _start: { uint8_t x_4; @@ -4261,13 +4387,13 @@ if (x_4 == 0) { lean_object* x_5; lean_object* x_6; uint8_t x_7; x_5 = lean_array_uget(x_1, x_2); -x_6 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__3; +x_6 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__3; lean_inc(x_5); x_7 = l_Lean_Syntax_isOfKind(x_5, x_6); if (x_7 == 0) { lean_object* x_8; uint8_t x_9; -x_8 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__5; +x_8 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__5; lean_inc(x_5); x_9 = l_Lean_Syntax_isOfKind(x_5, x_8); if (x_9 == 0) @@ -4284,7 +4410,7 @@ else lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; x_13 = lean_unsigned_to_nat(0u); x_14 = l_Lean_Syntax_getArg(x_5, x_13); -x_15 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__7; +x_15 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__7; x_16 = l_Lean_Syntax_matchesIdent(x_14, x_15); lean_dec(x_14); if (x_16 == 0) @@ -4336,7 +4462,7 @@ return x_28; } } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__1() { _start: { lean_object* x_1; @@ -4344,7 +4470,7 @@ x_1 = lean_mk_string_unchecked("Term", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__2() { _start: { lean_object* x_1; @@ -4352,19 +4478,19 @@ x_1 = lean_mk_string_unchecked("attrInstance", 12, 12); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__3() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__1; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__2; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__1; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__2; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__4() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__4() { _start: { lean_object* x_1; @@ -4372,23 +4498,23 @@ x_1 = lean_mk_string_unchecked("attrKind", 8, 8); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__5() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__1; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__4; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__1; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__4; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__3; lean_inc(x_1); x_3 = l_Lean_Syntax_isOfKind(x_1, x_2); if (x_3 == 0) @@ -4403,7 +4529,7 @@ else lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; x_5 = lean_unsigned_to_nat(0u); x_6 = l_Lean_Syntax_getArg(x_1, x_5); -x_7 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__5; +x_7 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__5; lean_inc(x_6); x_8 = l_Lean_Syntax_isOfKind(x_6, x_7); if (x_8 == 0) @@ -4441,7 +4567,7 @@ return x_15; } } } -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_5; lean_object* x_6; uint8_t x_7; @@ -4485,14 +4611,14 @@ size_t x_16; size_t x_17; uint8_t x_18; x_16 = 0; x_17 = lean_usize_of_nat(x_13); lean_dec(x_13); -x_18 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3(x_2, x_16, x_17); +x_18 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3(x_2, x_16, x_17); return x_18; } } } } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3___closed__1() { _start: { lean_object* x_1; @@ -4500,19 +4626,19 @@ x_1 = lean_mk_string_unchecked("noncomputable", 13, 13); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3___closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3___closed__1; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; uint8_t x_7; @@ -4538,7 +4664,7 @@ lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; x_11 = lean_unsigned_to_nat(0u); x_12 = l_Lean_Syntax_getArg(x_6, x_11); lean_dec(x_6); -x_13 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3___closed__2; +x_13 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3___closed__2; x_14 = l_Lean_Syntax_isOfKind(x_12, x_13); if (x_14 == 0) { @@ -4550,7 +4676,7 @@ else { lean_object* x_16; uint8_t x_17; x_16 = lean_box(0); -x_17 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__2(x_1, x_2, x_16); +x_17 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__2(x_1, x_2, x_16); return x_17; } } @@ -4560,12 +4686,12 @@ else lean_object* x_18; uint8_t x_19; lean_dec(x_6); x_18 = lean_box(0); -x_19 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__2(x_1, x_2, x_18); +x_19 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__2(x_1, x_2, x_18); return x_19; } } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__1() { _start: { lean_object* x_1; @@ -4573,19 +4699,19 @@ x_1 = lean_mk_string_unchecked("attributes", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__1; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__1; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__1; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__3() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__3() { _start: { lean_object* x_1; lean_object* x_2; @@ -4594,12 +4720,12 @@ x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__4() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__4() { _start: { uint8_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = 1; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__3; x_3 = lean_box(x_1); x_4 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_4, 0, x_3); @@ -4607,15 +4733,15 @@ lean_ctor_set(x_4, 1, x_2); return x_4; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__5() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__5() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1), 1, 0); return x_1; } } -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; lean_object* x_4; uint8_t x_5; @@ -4636,7 +4762,7 @@ lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; x_7 = lean_unsigned_to_nat(0u); x_8 = l_Lean_Syntax_getArg(x_4, x_7); lean_dec(x_4); -x_9 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__2; +x_9 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__2; lean_inc(x_8); x_10 = l_Lean_Syntax_isOfKind(x_8, x_9); if (x_10 == 0) @@ -4660,7 +4786,7 @@ if (x_15 == 0) lean_object* x_47; lean_dec(x_14); lean_dec(x_13); -x_47 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__3; +x_47 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__3; x_16 = x_47; goto block_46; } @@ -4673,7 +4799,7 @@ if (x_48 == 0) lean_object* x_49; lean_dec(x_14); lean_dec(x_13); -x_49 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__3; +x_49 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__3; x_16 = x_49; goto block_46; } @@ -4683,7 +4809,7 @@ size_t x_50; size_t x_51; lean_object* x_52; lean_object* x_53; lean_object* x_5 x_50 = 0; x_51 = lean_usize_of_nat(x_14); lean_dec(x_14); -x_52 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__4; +x_52 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__4; x_53 = l_Array_foldlMUnsafe_fold___at_Lean_Syntax_SepArray_getElems___spec__1(x_13, x_50, x_51, x_52); lean_dec(x_13); x_54 = lean_ctor_get(x_53, 1); @@ -4696,8 +4822,8 @@ goto block_46; block_46: { lean_object* x_17; lean_object* x_18; -x_17 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__5; -x_18 = l_Array_sequenceMap___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__1(x_16, x_17); +x_17 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__5; +x_18 = l_Array_sequenceMap___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__1(x_16, x_17); lean_dec(x_16); if (lean_obj_tag(x_18) == 0) { @@ -4737,7 +4863,7 @@ x_27 = l_Lean_Syntax_getArg(x_23, x_7); lean_dec(x_23); lean_ctor_set(x_18, 0, x_27); x_28 = lean_box(0); -x_29 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3(x_1, x_21, x_28, x_18); +x_29 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3(x_1, x_21, x_28, x_18); lean_dec(x_18); lean_dec(x_21); return x_29; @@ -4750,7 +4876,7 @@ lean_dec(x_23); lean_free_object(x_18); x_30 = lean_box(0); x_31 = lean_box(0); -x_32 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3(x_1, x_21, x_31, x_30); +x_32 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3(x_1, x_21, x_31, x_30); lean_dec(x_21); return x_32; } @@ -4785,7 +4911,7 @@ lean_dec(x_35); x_40 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_40, 0, x_39); x_41 = lean_box(0); -x_42 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3(x_1, x_33, x_41, x_40); +x_42 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3(x_1, x_33, x_41, x_40); lean_dec(x_40); lean_dec(x_33); return x_42; @@ -4797,7 +4923,7 @@ lean_object* x_43; lean_object* x_44; uint8_t x_45; lean_dec(x_35); x_43 = lean_box(0); x_44 = lean_box(0); -x_45 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3(x_1, x_33, x_44, x_43); +x_45 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3(x_1, x_33, x_44, x_43); lean_dec(x_33); return x_45; } @@ -4808,7 +4934,7 @@ return x_45; } } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__1() { _start: { lean_object* x_1; @@ -4816,19 +4942,19 @@ x_1 = lean_mk_string_unchecked("declModifiers", 13, 13); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__1; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__3() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__3() { _start: { lean_object* x_1; @@ -4836,19 +4962,19 @@ x_1 = lean_mk_string_unchecked("docComment", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__4() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__3; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__5() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__5() { _start: { lean_object* x_1; @@ -4856,105 +4982,105 @@ x_1 = lean_mk_string_unchecked("declaration", 11, 11); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__6() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__5; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__5; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__7() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__7() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__6; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__6; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__8() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__7; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__7; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__9() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__8; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__8; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__10() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__9; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__9; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__11() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__10; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__10; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__12() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__11; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__11; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__13() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__12; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__12; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_29; uint8_t x_30; -x_29 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__13; +x_29 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__13; lean_inc(x_2); x_30 = l_Lean_Syntax_Stack_matches(x_2, x_29); if (x_30 == 0) @@ -4985,13 +5111,13 @@ lean_dec(x_33); x_36 = lean_ctor_get(x_35, 0); lean_inc(x_36); lean_dec(x_35); -x_37 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__10; +x_37 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__10; lean_inc(x_36); x_38 = l_Lean_Syntax_isOfKind(x_36, x_37); if (x_38 == 0) { lean_object* x_39; uint8_t x_40; -x_39 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__12; +x_39 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__12; x_40 = l_Lean_Syntax_isOfKind(x_36, x_39); if (x_40 == 0) { @@ -5043,7 +5169,7 @@ lean_dec(x_8); x_10 = lean_unsigned_to_nat(0u); x_11 = l_Lean_Syntax_getArg(x_9, x_10); lean_dec(x_9); -x_12 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__2; +x_12 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__2; lean_inc(x_11); x_13 = l_Lean_Syntax_isOfKind(x_11, x_12); if (x_13 == 0) @@ -5077,7 +5203,7 @@ else lean_object* x_20; lean_object* x_21; uint8_t x_22; x_20 = l_Lean_Syntax_getArg(x_15, x_10); lean_dec(x_15); -x_21 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__4; +x_21 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__4; x_22 = l_Lean_Syntax_isOfKind(x_20, x_21); if (x_22 == 0) { @@ -5090,7 +5216,7 @@ else { lean_object* x_24; uint8_t x_25; x_24 = lean_box(0); -x_25 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4(x_11, x_24); +x_25 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4(x_11, x_24); lean_dec(x_11); return x_25; } @@ -5101,7 +5227,7 @@ else lean_object* x_26; uint8_t x_27; lean_dec(x_15); x_26 = lean_box(0); -x_27 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4(x_11, x_26); +x_27 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4(x_11, x_26); lean_dec(x_11); return x_27; } @@ -5110,42 +5236,42 @@ return x_27; } } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___boxed), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___boxed), 3, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____closed__1; x_3 = l_Lean_Linter_addBuiltinUnusedVariablesIgnoreFn(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Array_sequenceMap_loop___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Array_sequenceMap_loop___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; -x_6 = l_Array_sequenceMap_loop___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__2(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Array_sequenceMap_loop___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__2(x_1, x_2, x_3, x_4, x_5); lean_dec(x_1); return x_6; } } -LEAN_EXPORT lean_object* l_Array_sequenceMap___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__1___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_sequenceMap___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__1___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Array_sequenceMap___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__1(x_1, x_2); +x_3 = l_Array_sequenceMap___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__1(x_1, x_2); lean_dec(x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { size_t x_4; size_t x_5; uint8_t x_6; lean_object* x_7; @@ -5153,17 +5279,17 @@ x_4 = lean_unbox_usize(x_2); lean_dec(x_2); x_5 = lean_unbox_usize(x_3); lean_dec(x_3); -x_6 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3(x_1, x_4, x_5); +x_6 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3(x_1, x_4, x_5); lean_dec(x_1); x_7 = lean_box(x_6); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__2(x_1, x_2, x_3); +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__2(x_1, x_2, x_3); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); @@ -5171,11 +5297,11 @@ x_5 = lean_box(x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { uint8_t x_5; lean_object* x_6; -x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3(x_1, x_2, x_3, x_4); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); @@ -5184,29 +5310,29 @@ x_6 = lean_box(x_5); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4(x_1, x_2); +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4(x_1, x_2); lean_dec(x_2); lean_dec(x_1); x_4 = lean_box(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5(x_1, x_2, x_3); +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5(x_1, x_2, x_3); lean_dec(x_3); lean_dec(x_1); x_5 = lean_box(x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__1() { _start: { lean_object* x_1; @@ -5214,29 +5340,29 @@ x_1 = lean_mk_string_unchecked("explicitBinder", 14, 14); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__1; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__1; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__1; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__3() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__2; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__2; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__4() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__4() { _start: { lean_object* x_1; @@ -5244,102 +5370,102 @@ x_1 = lean_mk_string_unchecked("depArrow", 8, 8); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__5() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__1; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__4; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__1; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__4; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__6() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__6() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__5; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__5; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__7() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__6; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__6; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__8() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__7; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__7; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__9() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__8; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__8; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; uint8_t x_5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__9; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__9; x_5 = l_Lean_Syntax_Stack_matches(x_2, x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___boxed), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___boxed), 3, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____closed__1; x_3 = l_Lean_Linter_addBuiltinUnusedVariablesIgnoreFn(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1(x_1, x_2, x_3); +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1(x_1, x_2, x_3); lean_dec(x_3); lean_dec(x_1); x_5 = lean_box(x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__1() { _start: { lean_object* x_1; @@ -5347,77 +5473,77 @@ x_1 = lean_mk_string_unchecked("letIdDecl", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__1; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__1; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__1; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__3() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__2; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__2; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__4() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__2; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__2; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__5() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__4; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__4; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__6() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__5; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__5; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__7() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__6; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__6; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__8() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__8() { _start: { lean_object* x_1; @@ -5425,19 +5551,19 @@ x_1 = lean_mk_string_unchecked("whereStructField", 16, 16); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__9() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__8; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__8; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -5445,7 +5571,7 @@ x_4 = l_Lean_Linter_getLinterUnusedVariablesFunArgs(x_3); if (x_4 == 0) { lean_object* x_5; uint8_t x_6; -x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__7; +x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__7; lean_inc(x_2); x_6 = l_Lean_Syntax_Stack_matches(x_2, x_5); if (x_6 == 0) @@ -5507,7 +5633,7 @@ lean_dec(x_17); x_20 = lean_ctor_get(x_19, 0); lean_inc(x_20); lean_dec(x_19); -x_21 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__9; +x_21 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__9; x_22 = l_Lean_Syntax_isOfKind(x_20, x_21); if (x_22 == 0) { @@ -5535,71 +5661,71 @@ return x_25; } } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___boxed), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___boxed), 3, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____closed__1; x_3 = l_Lean_Linter_addBuiltinUnusedVariablesIgnoreFn(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1(x_1, x_2, x_3); +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1(x_1, x_2, x_3); lean_dec(x_3); lean_dec(x_1); x_5 = lean_box(x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__2; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__2; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__1; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__3() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__2; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__2; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -5607,7 +5733,7 @@ x_4 = l_Lean_Linter_getLinterUnusedVariablesFunArgs(x_3); if (x_4 == 0) { lean_object* x_5; uint8_t x_6; -x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__3; +x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__3; lean_inc(x_2); x_6 = l_Lean_Syntax_Stack_matches(x_2, x_5); if (x_6 == 0) @@ -5655,7 +5781,7 @@ else lean_object* x_17; lean_object* x_18; uint8_t x_19; x_17 = lean_alloc_closure((void*)(l_Lean_Syntax_isOfKind___boxed), 2, 1); lean_closure_set(x_17, 0, x_12); -x_18 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__14; +x_18 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__14; x_19 = l_List_any___rarg(x_18, x_17); return x_19; } @@ -5671,35 +5797,35 @@ return x_20; } } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___boxed), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___boxed), 3, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____closed__1; x_3 = l_Lean_Linter_addBuiltinUnusedVariablesIgnoreFn(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1(x_1, x_2, x_3); +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1(x_1, x_2, x_3); lean_dec(x_3); lean_dec(x_1); x_5 = lean_box(x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__1() { _start: { lean_object* x_1; @@ -5707,53 +5833,53 @@ x_1 = lean_mk_string_unchecked("basicFun", 8, 8); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__1; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__1; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__1; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__3() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__2; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__2; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__4() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__3; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__5() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__4; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__4; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__6() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__6() { _start: { lean_object* x_1; @@ -5761,41 +5887,41 @@ x_1 = lean_mk_string_unchecked("typeAscription", 14, 14); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__7() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__1; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__6; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__1; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__6; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__8() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__8() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__7; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__7; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__9() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__8; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__5; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__8; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__5; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -5803,13 +5929,13 @@ x_4 = l_Lean_Linter_getLinterUnusedVariablesFunArgs(x_3); if (x_4 == 0) { lean_object* x_5; uint8_t x_6; -x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__5; +x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__5; lean_inc(x_2); x_6 = l_Lean_Syntax_Stack_matches(x_2, x_5); if (x_6 == 0) { lean_object* x_7; uint8_t x_8; -x_7 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__9; +x_7 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__9; x_8 = l_Lean_Syntax_Stack_matches(x_2, x_7); return x_8; } @@ -5830,35 +5956,35 @@ return x_10; } } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___boxed), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___boxed), 3, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____closed__1; x_3 = l_Lean_Linter_addBuiltinUnusedVariablesIgnoreFn(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1(x_1, x_2, x_3); +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1(x_1, x_2, x_3); lean_dec(x_3); lean_dec(x_1); x_5 = lean_box(x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__1() { _start: { lean_object* x_1; @@ -5866,19 +5992,19 @@ x_1 = lean_mk_string_unchecked("matchAlt", 8, 8); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__1; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__1; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__1; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__3() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__3() { _start: { lean_object* x_1; @@ -5886,7 +6012,7 @@ x_1 = lean_mk_string_unchecked("Tactic", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__4() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__4() { _start: { lean_object* x_1; @@ -5894,19 +6020,19 @@ x_1 = lean_mk_string_unchecked("inductionAltLHS", 15, 15); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__5() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__3; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__4; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__3; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__4; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1(lean_object* x_1) { +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; uint8_t x_5; @@ -5915,13 +6041,13 @@ lean_inc(x_2); x_3 = lean_ctor_get(x_1, 1); lean_inc(x_3); lean_dec(x_1); -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__2; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__2; lean_inc(x_2); x_5 = l_Lean_Syntax_isOfKind(x_2, x_4); if (x_5 == 0) { lean_object* x_6; uint8_t x_7; -x_6 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__5; +x_6 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__5; x_7 = l_Lean_Syntax_isOfKind(x_2, x_6); if (x_7 == 0) { @@ -5947,7 +6073,7 @@ x_12 = lean_nat_dec_eq(x_3, x_11); if (x_12 == 0) { lean_object* x_13; uint8_t x_14; -x_13 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__5; +x_13 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__5; x_14 = l_Lean_Syntax_isOfKind(x_2, x_13); if (x_14 == 0) { @@ -5976,15 +6102,15 @@ return x_18; } } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__2___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__2___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___boxed), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___boxed), 1, 0); return x_1; } } -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -5992,7 +6118,7 @@ x_4 = l_Lean_Linter_getLinterUnusedVariablesPatternVars(x_3); if (x_4 == 0) { lean_object* x_5; uint8_t x_6; -x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__2___closed__1; +x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__2___closed__1; x_6 = l_List_any___rarg(x_2, x_5); return x_6; } @@ -6005,37 +6131,37 @@ return x_7; } } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__2___boxed), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__2___boxed), 3, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____closed__1; x_3 = l_Lean_Linter_addBuiltinUnusedVariablesIgnoreFn(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___boxed(lean_object* x_1) { _start: { uint8_t x_2; lean_object* x_3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1(x_1); +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1(x_1); x_3 = lean_box(x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__2(x_1, x_2, x_3); +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__2(x_1, x_2, x_3); lean_dec(x_3); lean_dec(x_1); x_5 = lean_box(x_4); @@ -6047,7 +6173,7 @@ static lean_object* _init_l_Lean_Linter_getUnusedVariablesIgnoreFns___rarg___clo { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__3; x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); @@ -6068,7 +6194,7 @@ x_6 = lean_ctor_get(x_5, 0); lean_inc(x_6); lean_dec(x_5); x_7 = l_Lean_Linter_getUnusedVariablesIgnoreFns___rarg___closed__1; -x_8 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__5___closed__1; +x_8 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__5___closed__1; x_9 = l_Lean_PersistentEnvExtension_getState___rarg(x_7, x_8, x_6); lean_dec(x_6); x_10 = lean_ctor_get(x_9, 1); @@ -6089,7 +6215,7 @@ x_13 = lean_ctor_get(x_11, 0); lean_inc(x_13); lean_dec(x_11); x_14 = l_Lean_Linter_getUnusedVariablesIgnoreFns___rarg___closed__1; -x_15 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__5___closed__1; +x_15 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__5___closed__1; x_16 = l_Lean_PersistentEnvExtension_getState___rarg(x_14, x_15, x_13); lean_dec(x_13); x_17 = lean_ctor_get(x_16, 1); @@ -9316,8 +9442,8 @@ static lean_object* _init_l_Lean_Linter_UnusedVariables_collectReferences_skipDe { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5; x_4 = l_Lean_Linter_UnusedVariables_collectReferences_skipDeclIdIfPresent___closed__1; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; @@ -9344,7 +9470,7 @@ return x_5; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_collectReferences___spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__1(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -9376,7 +9502,7 @@ return x_9; } } } -LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__2(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__2(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -9405,7 +9531,7 @@ return x_8; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_collectReferences___spec__5(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__5(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -9479,7 +9605,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; uint8_t x_5; @@ -9498,7 +9624,7 @@ lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_obj x_6 = lean_array_fget(x_2, x_1); x_7 = lean_box(0); x_8 = lean_array_fset(x_2, x_1, x_7); -x_9 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_collectReferences___spec__5(x_3, x_6); +x_9 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__5(x_3, x_6); x_10 = lean_unsigned_to_nat(1u); x_11 = lean_nat_add(x_1, x_10); lean_dec(x_1); @@ -9509,7 +9635,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__3(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__3(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; @@ -9520,11 +9646,11 @@ lean_dec(x_2); x_5 = lean_box(0); x_6 = lean_mk_array(x_4, x_5); x_7 = lean_unsigned_to_nat(0u); -x_8 = l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__4(x_7, x_1, x_6); +x_8 = l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__4(x_7, x_1, x_6); return x_8; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_3) == 0) @@ -9549,7 +9675,7 @@ x_9 = l___private_Lean_Syntax_0__String_beqRange____x40_Lean_Syntax___hyg_95_(x_ if (x_9 == 0) { lean_object* x_10; -x_10 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__6(x_1, x_2, x_8); +x_10 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__6(x_1, x_2, x_8); lean_ctor_set(x_3, 2, x_10); return x_3; } @@ -9576,7 +9702,7 @@ x_14 = l___private_Lean_Syntax_0__String_beqRange____x40_Lean_Syntax___hyg_95_(x if (x_14 == 0) { lean_object* x_15; lean_object* x_16; -x_15 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__6(x_1, x_2, x_13); +x_15 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__6(x_1, x_2, x_13); x_16 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_16, 0, x_11); lean_ctor_set(x_16, 1, x_12); @@ -9598,7 +9724,7 @@ return x_17; } } } -LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__7(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__7(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -9627,7 +9753,7 @@ return x_8; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_collectReferences___spec__10(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__10(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -9701,7 +9827,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; uint8_t x_5; @@ -9720,7 +9846,7 @@ lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_obj x_6 = lean_array_fget(x_2, x_1); x_7 = lean_box(0); x_8 = lean_array_fset(x_2, x_1, x_7); -x_9 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_collectReferences___spec__10(x_3, x_6); +x_9 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__10(x_3, x_6); x_10 = lean_unsigned_to_nat(1u); x_11 = lean_nat_add(x_1, x_10); lean_dec(x_1); @@ -9731,7 +9857,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__8(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__8(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; @@ -9742,11 +9868,194 @@ lean_dec(x_2); x_5 = lean_box(0); x_6 = lean_mk_array(x_4, x_5); x_7 = lean_unsigned_to_nat(0u); -x_8 = l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__9(x_7, x_1, x_6); +x_8 = l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__9(x_7, x_1, x_6); +return x_8; +} +} +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__13(lean_object* x_1, size_t x_2, size_t x_3) { +_start: +{ +uint8_t x_4; +x_4 = lean_usize_dec_eq(x_2, x_3); +if (x_4 == 0) +{ +lean_object* x_5; uint8_t x_6; +x_5 = lean_array_uget(x_1, x_2); +x_6 = l_Lean_PersistentArray_anyMAux___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__12(x_5); +lean_dec(x_5); +if (x_6 == 0) +{ +size_t x_7; size_t x_8; +x_7 = 1; +x_8 = lean_usize_add(x_2, x_7); +x_2 = x_8; +goto _start; +} +else +{ +uint8_t x_10; +x_10 = 1; +return x_10; +} +} +else +{ +uint8_t x_11; +x_11 = 0; +return x_11; +} +} +} +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14___lambda__1(lean_object* x_1) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +uint8_t x_2; +x_2 = 1; +return x_2; +} +else +{ +uint8_t x_3; +x_3 = 0; +return x_3; +} +} +} +static lean_object* _init_l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14___lambda__1___boxed), 1, 0); +return x_1; +} +} +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14(lean_object* x_1, size_t x_2, size_t x_3) { +_start: +{ +uint8_t x_4; +x_4 = lean_usize_dec_eq(x_2, x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_5 = lean_array_uget(x_1, x_2); +x_6 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14___closed__1; +x_7 = l_Lean_Elab_InfoTree_findInfo_x3f(x_6, x_5); +if (lean_obj_tag(x_7) == 0) +{ +size_t x_8; size_t x_9; +x_8 = 1; +x_9 = lean_usize_add(x_2, x_8); +x_2 = x_9; +goto _start; +} +else +{ +uint8_t x_11; +lean_dec(x_7); +x_11 = 1; +return x_11; +} +} +else +{ +uint8_t x_12; +x_12 = 0; +return x_12; +} +} +} +LEAN_EXPORT uint8_t l_Lean_PersistentArray_anyMAux___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__12(lean_object* x_1) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; uint8_t x_5; +x_2 = lean_ctor_get(x_1, 0); +x_3 = lean_array_get_size(x_2); +x_4 = lean_unsigned_to_nat(0u); +x_5 = lean_nat_dec_lt(x_4, x_3); +if (x_5 == 0) +{ +uint8_t x_6; +lean_dec(x_3); +x_6 = 0; +return x_6; +} +else +{ +size_t x_7; size_t x_8; uint8_t x_9; +x_7 = 0; +x_8 = lean_usize_of_nat(x_3); +lean_dec(x_3); +x_9 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__13(x_2, x_7, x_8); +return x_9; +} +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_10 = lean_ctor_get(x_1, 0); +x_11 = lean_array_get_size(x_10); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_nat_dec_lt(x_12, x_11); +if (x_13 == 0) +{ +uint8_t x_14; +lean_dec(x_11); +x_14 = 0; +return x_14; +} +else +{ +size_t x_15; size_t x_16; uint8_t x_17; +x_15 = 0; +x_16 = lean_usize_of_nat(x_11); +lean_dec(x_11); +x_17 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14(x_10, x_15, x_16); +return x_17; +} +} +} +} +LEAN_EXPORT uint8_t l_Lean_PersistentArray_anyM___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__11(lean_object* x_1) { +_start: +{ +lean_object* x_2; uint8_t x_3; +x_2 = lean_ctor_get(x_1, 0); +x_3 = l_Lean_PersistentArray_anyMAux___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__12(x_2); +if (x_3 == 0) +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; uint8_t x_7; +x_4 = lean_ctor_get(x_1, 1); +x_5 = lean_array_get_size(x_4); +x_6 = lean_unsigned_to_nat(0u); +x_7 = lean_nat_dec_lt(x_6, x_5); +if (x_7 == 0) +{ +uint8_t x_8; +lean_dec(x_5); +x_8 = 0; return x_8; } +else +{ +size_t x_9; size_t x_10; uint8_t x_11; +x_9 = 0; +x_10 = lean_usize_of_nat(x_5); +lean_dec(x_5); +x_11 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14(x_4, x_9, x_10); +return x_11; +} +} +else +{ +return x_3; +} +} } -LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__11(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__15(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -9775,7 +10084,7 @@ return x_8; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_collectReferences___spec__14(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__18(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -9849,7 +10158,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__13(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__17(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; uint8_t x_5; @@ -9868,7 +10177,7 @@ lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_obj x_6 = lean_array_fget(x_2, x_1); x_7 = lean_box(0); x_8 = lean_array_fset(x_2, x_1, x_7); -x_9 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_collectReferences___spec__14(x_3, x_6); +x_9 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__18(x_3, x_6); x_10 = lean_unsigned_to_nat(1u); x_11 = lean_nat_add(x_1, x_10); lean_dec(x_1); @@ -9879,7 +10188,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__12(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__16(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; @@ -9890,11 +10199,11 @@ lean_dec(x_2); x_5 = lean_box(0); x_6 = lean_mk_array(x_4, x_5); x_7 = lean_unsigned_to_nat(0u); -x_8 = l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__13(x_7, x_1, x_6); +x_8 = l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__17(x_7, x_1, x_6); return x_8; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__15(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__19(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_3) == 0) @@ -9919,7 +10228,7 @@ x_9 = lean_name_eq(x_6, x_1); if (x_9 == 0) { lean_object* x_10; -x_10 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__15(x_1, x_2, x_8); +x_10 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__19(x_1, x_2, x_8); lean_ctor_set(x_3, 2, x_10); return x_3; } @@ -9946,7 +10255,7 @@ x_14 = lean_name_eq(x_11, x_1); if (x_14 == 0) { lean_object* x_15; lean_object* x_16; -x_15 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__15(x_1, x_2, x_13); +x_15 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__19(x_1, x_2, x_13); x_16 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_16, 0, x_11); lean_ctor_set(x_16, 1, x_12); @@ -9968,7 +10277,7 @@ return x_17; } } } -static lean_object* _init_l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__1() { +static lean_object* _init_l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__1() { _start: { lean_object* x_1; @@ -9976,179 +10285,189 @@ x_1 = l_EStateM_instMonad(lean_box(0), lean_box(0)); return x_1; } } -static lean_object* _init_l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__2() { +static lean_object* _init_l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__1; +x_2 = l_ReaderT_instMonad___rarg(x_1); +return x_2; +} +} +static lean_object* _init_l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__1; +x_1 = l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__2; x_2 = l_ReaderT_instMonad___rarg(x_1); return x_2; } } -static lean_object* _init_l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__3() { +static lean_object* _init_l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__2; +x_2 = l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__3; x_3 = l_instInhabitedOfMonad___rarg(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_4 = l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__3; -x_5 = lean_panic_fn(x_4, x_1); -x_6 = lean_apply_2(x_5, x_2, x_3); -return x_6; +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__4; +x_6 = lean_panic_fn(x_5, x_1); +x_7 = lean_box(x_2); +x_8 = lean_apply_3(x_6, x_7, x_3, x_4); +return x_8; } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__20(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__23(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8) { _start: { if (lean_obj_tag(x_4) == 0) { -lean_object* x_8; lean_object* x_9; -lean_dec(x_6); +lean_object* x_9; lean_object* x_10; +lean_dec(x_7); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_8 = l_List_reverse___rarg(x_5); -x_9 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_9, 0, x_8); -lean_ctor_set(x_9, 1, x_7); -return x_9; +x_9 = l_List_reverse___rarg(x_5); +x_10 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set(x_10, 1, x_8); +return x_10; } else { -uint8_t x_10; -x_10 = !lean_is_exclusive(x_4); -if (x_10 == 0) +uint8_t x_11; +x_11 = !lean_is_exclusive(x_4); +if (x_11 == 0) { -lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_11 = lean_ctor_get(x_4, 0); -x_12 = lean_ctor_get(x_4, 1); -lean_inc(x_6); +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_4, 0); +x_13 = lean_ctor_get(x_4, 1); +lean_inc(x_7); lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_13 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18(x_1, x_2, x_3, x_11, x_6, x_7); -if (lean_obj_tag(x_13) == 0) +x_14 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21(x_1, x_2, x_3, x_12, x_6, x_7, x_8); +if (lean_obj_tag(x_14) == 0) { -lean_object* x_14; lean_object* x_15; -x_14 = lean_ctor_get(x_13, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_13, 1); +lean_object* x_15; lean_object* x_16; +x_15 = lean_ctor_get(x_14, 0); lean_inc(x_15); -lean_dec(x_13); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); lean_ctor_set(x_4, 1, x_5); -lean_ctor_set(x_4, 0, x_14); +lean_ctor_set(x_4, 0, x_15); { -lean_object* _tmp_3 = x_12; +lean_object* _tmp_3 = x_13; lean_object* _tmp_4 = x_4; -lean_object* _tmp_6 = x_15; +lean_object* _tmp_7 = x_16; x_4 = _tmp_3; x_5 = _tmp_4; -x_7 = _tmp_6; +x_8 = _tmp_7; } goto _start; } else { -uint8_t x_17; +uint8_t x_18; lean_free_object(x_4); -lean_dec(x_12); -lean_dec(x_6); -lean_dec(x_5); +lean_dec(x_13); +lean_dec(x_7); +lean_dec(x_5); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_17 = !lean_is_exclusive(x_13); -if (x_17 == 0) +x_18 = !lean_is_exclusive(x_14); +if (x_18 == 0) { -return x_13; +return x_14; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_13, 0); -x_19 = lean_ctor_get(x_13, 1); +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_14, 0); +x_20 = lean_ctor_get(x_14, 1); +lean_inc(x_20); lean_inc(x_19); -lean_inc(x_18); -lean_dec(x_13); -x_20 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_20, 0, x_18); -lean_ctor_set(x_20, 1, x_19); -return x_20; +lean_dec(x_14); +x_21 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_21, 0, x_19); +lean_ctor_set(x_21, 1, x_20); +return x_21; } } } else { -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_4, 0); -x_22 = lean_ctor_get(x_4, 1); +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_4, 0); +x_23 = lean_ctor_get(x_4, 1); +lean_inc(x_23); lean_inc(x_22); -lean_inc(x_21); lean_dec(x_4); -lean_inc(x_6); +lean_inc(x_7); lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_23 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18(x_1, x_2, x_3, x_21, x_6, x_7); -if (lean_obj_tag(x_23) == 0) +x_24 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21(x_1, x_2, x_3, x_22, x_6, x_7, x_8); +if (lean_obj_tag(x_24) == 0) { -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_23, 1); +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_24, 0); lean_inc(x_25); -lean_dec(x_23); -x_26 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_26, 0, x_24); -lean_ctor_set(x_26, 1, x_5); -x_4 = x_22; -x_5 = x_26; -x_7 = x_25; +x_26 = lean_ctor_get(x_24, 1); +lean_inc(x_26); +lean_dec(x_24); +x_27 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_5); +x_4 = x_23; +x_5 = x_27; +x_8 = x_26; goto _start; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; -lean_dec(x_22); -lean_dec(x_6); +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +lean_dec(x_23); +lean_dec(x_7); lean_dec(x_5); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_28 = lean_ctor_get(x_23, 0); -lean_inc(x_28); -x_29 = lean_ctor_get(x_23, 1); +x_29 = lean_ctor_get(x_24, 0); lean_inc(x_29); -if (lean_is_exclusive(x_23)) { - lean_ctor_release(x_23, 0); - lean_ctor_release(x_23, 1); - x_30 = x_23; +x_30 = lean_ctor_get(x_24, 1); +lean_inc(x_30); +if (lean_is_exclusive(x_24)) { + lean_ctor_release(x_24, 0); + lean_ctor_release(x_24, 1); + x_31 = x_24; } else { - lean_dec_ref(x_23); - x_30 = lean_box(0); + lean_dec_ref(x_24); + x_31 = lean_box(0); } -if (lean_is_scalar(x_30)) { - x_31 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_31)) { + x_32 = lean_alloc_ctor(1, 2, 0); } else { - x_31 = x_30; + x_32 = x_31; } -lean_ctor_set(x_31, 0, x_28); -lean_ctor_set(x_31, 1, x_29); -return x_31; +lean_ctor_set(x_32, 0, x_29); +lean_ctor_set(x_32, 1, x_30); +return x_32; } } } } } -static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__1() { +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__1() { _start: { lean_object* x_1; @@ -10156,7 +10475,7 @@ x_1 = lean_mk_string_unchecked("Lean.Server.InfoUtils", 21, 21); return x_1; } } -static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__2() { +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__2() { _start: { lean_object* x_1; @@ -10164,7 +10483,7 @@ x_1 = lean_mk_string_unchecked("Lean.Elab.InfoTree.visitM.go", 28, 28); return x_1; } } -static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__3() { +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__3() { _start: { lean_object* x_1; @@ -10172,20 +10491,20 @@ x_1 = lean_mk_string_unchecked("unexpected context-free info tree node", 38, 38) return x_1; } } -static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__4() { +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__1; -x_2 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__2; -x_3 = lean_unsigned_to_nat(56u); +x_1 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__1; +x_2 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__2; +x_3 = lean_unsigned_to_nat(62u); x_4 = lean_unsigned_to_nat(21u); -x_5 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__3; +x_5 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, lean_object* x_6, lean_object* x_7) { _start: { if (lean_obj_tag(x_3) == 0) @@ -10193,39 +10512,39 @@ if (lean_obj_tag(x_3) == 0) switch (lean_obj_tag(x_4)) { case 0: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; -x_7 = lean_ctor_get(x_4, 0); -lean_inc(x_7); -x_8 = lean_ctor_get(x_4, 1); +lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_8 = lean_ctor_get(x_4, 0); lean_inc(x_8); +x_9 = lean_ctor_get(x_4, 1); +lean_inc(x_9); lean_dec(x_4); -x_9 = l_Lean_Elab_PartialContextInfo_mergeIntoOuter_x3f(x_7, x_3); -x_3 = x_9; -x_4 = x_8; +x_10 = l_Lean_Elab_PartialContextInfo_mergeIntoOuter_x3f(x_8, x_3); +x_3 = x_10; +x_4 = x_9; goto _start; } case 1: { -lean_object* x_11; lean_object* x_12; +lean_object* x_12; lean_object* x_13; lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_11 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__4; -x_12 = l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19(x_11, x_5, x_6); -return x_12; +x_12 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__4; +x_13 = l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22(x_12, x_5, x_6, x_7); +return x_13; } default: { -lean_object* x_13; lean_object* x_14; -lean_dec(x_5); +lean_object* x_14; lean_object* x_15; +lean_dec(x_6); lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_13 = lean_box(0); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_13); -lean_ctor_set(x_14, 1, x_6); -return x_14; +x_14 = lean_box(0); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_7); +return x_15; } } } @@ -10234,554 +10553,766 @@ else switch (lean_obj_tag(x_4)) { case 0: { -lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = lean_ctor_get(x_4, 0); -lean_inc(x_15); -x_16 = lean_ctor_get(x_4, 1); +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_4, 0); lean_inc(x_16); +x_17 = lean_ctor_get(x_4, 1); +lean_inc(x_17); lean_dec(x_4); -x_17 = l_Lean_Elab_PartialContextInfo_mergeIntoOuter_x3f(x_15, x_3); -x_3 = x_17; -x_4 = x_16; +x_18 = l_Lean_Elab_PartialContextInfo_mergeIntoOuter_x3f(x_16, x_3); +x_3 = x_18; +x_4 = x_17; goto _start; } case 1: { -uint8_t x_19; -x_19 = !lean_is_exclusive(x_3); -if (x_19 == 0) +uint8_t x_20; +x_20 = !lean_is_exclusive(x_3); +if (x_20 == 0) { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_20 = lean_ctor_get(x_3, 0); -x_21 = lean_ctor_get(x_4, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_4, 1); +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_21 = lean_ctor_get(x_3, 0); +x_22 = lean_ctor_get(x_4, 0); lean_inc(x_22); +x_23 = lean_ctor_get(x_4, 1); +lean_inc(x_23); lean_dec(x_4); +x_24 = lean_box(x_5); lean_inc(x_1); -lean_inc(x_5); +lean_inc(x_6); +lean_inc(x_23); lean_inc(x_22); lean_inc(x_21); -lean_inc(x_20); -x_23 = lean_apply_5(x_1, x_20, x_21, x_22, x_5, x_6); -if (lean_obj_tag(x_23) == 0) +x_25 = lean_apply_6(x_1, x_21, x_22, x_23, x_24, x_6, x_7); +if (lean_obj_tag(x_25) == 0) { -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_24 = lean_ctor_get(x_23, 1); -lean_inc(x_24); -lean_dec(x_23); -lean_inc(x_20); -x_25 = l_Lean_Elab_Info_updateContext_x3f(x_3, x_21); -x_26 = l_Lean_PersistentArray_toList___rarg(x_22); -x_27 = lean_box(0); -lean_inc(x_5); -lean_inc(x_2); -x_28 = l_List_mapM_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__20(x_1, x_2, x_25, x_26, x_27, x_5, x_24); -if (lean_obj_tag(x_28) == 0) +lean_object* x_26; uint8_t x_27; +x_26 = lean_ctor_get(x_25, 0); +lean_inc(x_26); +x_27 = lean_unbox(x_26); +lean_dec(x_26); +if (x_27 == 0) { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_28, 0); -lean_inc(x_29); -x_30 = lean_ctor_get(x_28, 1); -lean_inc(x_30); -lean_dec(x_28); -x_31 = lean_apply_6(x_2, x_20, x_21, x_22, x_29, x_5, x_30); +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +lean_dec(x_1); +x_28 = lean_ctor_get(x_25, 1); +lean_inc(x_28); +lean_dec(x_25); +x_29 = lean_box(0); +x_30 = lean_box(x_5); +x_31 = lean_apply_7(x_2, x_21, x_22, x_23, x_29, x_30, x_6, x_28); if (lean_obj_tag(x_31) == 0) { uint8_t x_32; x_32 = !lean_is_exclusive(x_31); if (x_32 == 0) { -lean_object* x_33; lean_object* x_34; +lean_object* x_33; x_33 = lean_ctor_get(x_31, 0); -x_34 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_34, 0, x_33); -lean_ctor_set(x_31, 0, x_34); +lean_ctor_set(x_3, 0, x_33); +lean_ctor_set(x_31, 0, x_3); return x_31; } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_35 = lean_ctor_get(x_31, 0); -x_36 = lean_ctor_get(x_31, 1); -lean_inc(x_36); +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_31, 0); +x_35 = lean_ctor_get(x_31, 1); lean_inc(x_35); +lean_inc(x_34); lean_dec(x_31); -x_37 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_37, 0, x_35); -x_38 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_38, 0, x_37); -lean_ctor_set(x_38, 1, x_36); -return x_38; +lean_ctor_set(x_3, 0, x_34); +x_36 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_36, 0, x_3); +lean_ctor_set(x_36, 1, x_35); +return x_36; } } else { -uint8_t x_39; -x_39 = !lean_is_exclusive(x_31); -if (x_39 == 0) +uint8_t x_37; +lean_free_object(x_3); +x_37 = !lean_is_exclusive(x_31); +if (x_37 == 0) { return x_31; } else { -lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_40 = lean_ctor_get(x_31, 0); -x_41 = lean_ctor_get(x_31, 1); -lean_inc(x_41); -lean_inc(x_40); +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_31, 0); +x_39 = lean_ctor_get(x_31, 1); +lean_inc(x_39); +lean_inc(x_38); lean_dec(x_31); -x_42 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_42, 0, x_40); -lean_ctor_set(x_42, 1, x_41); -return x_42; +x_40 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +return x_40; +} +} +} +else +{ +lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_41 = lean_ctor_get(x_25, 1); +lean_inc(x_41); +lean_dec(x_25); +lean_inc(x_21); +x_42 = l_Lean_Elab_Info_updateContext_x3f(x_3, x_22); +x_43 = l_Lean_PersistentArray_toList___rarg(x_23); +x_44 = lean_box(0); +lean_inc(x_6); +lean_inc(x_2); +x_45 = l_List_mapM_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__23(x_1, x_2, x_42, x_43, x_44, x_5, x_6, x_41); +if (lean_obj_tag(x_45) == 0) +{ +lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_46 = lean_ctor_get(x_45, 0); +lean_inc(x_46); +x_47 = lean_ctor_get(x_45, 1); +lean_inc(x_47); +lean_dec(x_45); +x_48 = lean_box(x_5); +x_49 = lean_apply_7(x_2, x_21, x_22, x_23, x_46, x_48, x_6, x_47); +if (lean_obj_tag(x_49) == 0) +{ +uint8_t x_50; +x_50 = !lean_is_exclusive(x_49); +if (x_50 == 0) +{ +lean_object* x_51; lean_object* x_52; +x_51 = lean_ctor_get(x_49, 0); +x_52 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_52, 0, x_51); +lean_ctor_set(x_49, 0, x_52); +return x_49; +} +else +{ +lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; +x_53 = lean_ctor_get(x_49, 0); +x_54 = lean_ctor_get(x_49, 1); +lean_inc(x_54); +lean_inc(x_53); +lean_dec(x_49); +x_55 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_55, 0, x_53); +x_56 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_56, 0, x_55); +lean_ctor_set(x_56, 1, x_54); +return x_56; +} +} +else +{ +uint8_t x_57; +x_57 = !lean_is_exclusive(x_49); +if (x_57 == 0) +{ +return x_49; +} +else +{ +lean_object* x_58; lean_object* x_59; lean_object* x_60; +x_58 = lean_ctor_get(x_49, 0); +x_59 = lean_ctor_get(x_49, 1); +lean_inc(x_59); +lean_inc(x_58); +lean_dec(x_49); +x_60 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_60, 0, x_58); +lean_ctor_set(x_60, 1, x_59); +return x_60; } } } else { -uint8_t x_43; +uint8_t x_61; +lean_dec(x_23); lean_dec(x_22); lean_dec(x_21); -lean_dec(x_20); -lean_dec(x_5); +lean_dec(x_6); lean_dec(x_2); -x_43 = !lean_is_exclusive(x_28); -if (x_43 == 0) +x_61 = !lean_is_exclusive(x_45); +if (x_61 == 0) { -return x_28; +return x_45; } else { -lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_44 = lean_ctor_get(x_28, 0); -x_45 = lean_ctor_get(x_28, 1); -lean_inc(x_45); -lean_inc(x_44); -lean_dec(x_28); -x_46 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_46, 0, x_44); -lean_ctor_set(x_46, 1, x_45); -return x_46; +lean_object* x_62; lean_object* x_63; lean_object* x_64; +x_62 = lean_ctor_get(x_45, 0); +x_63 = lean_ctor_get(x_45, 1); +lean_inc(x_63); +lean_inc(x_62); +lean_dec(x_45); +x_64 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_64, 0, x_62); +lean_ctor_set(x_64, 1, x_63); +return x_64; +} } } } else { -uint8_t x_47; +uint8_t x_65; +lean_dec(x_23); lean_dec(x_22); -lean_dec(x_21); lean_free_object(x_3); -lean_dec(x_20); -lean_dec(x_5); +lean_dec(x_21); +lean_dec(x_6); lean_dec(x_2); lean_dec(x_1); -x_47 = !lean_is_exclusive(x_23); -if (x_47 == 0) +x_65 = !lean_is_exclusive(x_25); +if (x_65 == 0) { -return x_23; +return x_25; } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_ctor_get(x_23, 0); -x_49 = lean_ctor_get(x_23, 1); -lean_inc(x_49); -lean_inc(x_48); -lean_dec(x_23); -x_50 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_50, 0, x_48); -lean_ctor_set(x_50, 1, x_49); -return x_50; +lean_object* x_66; lean_object* x_67; lean_object* x_68; +x_66 = lean_ctor_get(x_25, 0); +x_67 = lean_ctor_get(x_25, 1); +lean_inc(x_67); +lean_inc(x_66); +lean_dec(x_25); +x_68 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_68, 0, x_66); +lean_ctor_set(x_68, 1, x_67); +return x_68; } } } else { -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; -x_51 = lean_ctor_get(x_3, 0); -lean_inc(x_51); +lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; +x_69 = lean_ctor_get(x_3, 0); +lean_inc(x_69); lean_dec(x_3); -x_52 = lean_ctor_get(x_4, 0); -lean_inc(x_52); -x_53 = lean_ctor_get(x_4, 1); -lean_inc(x_53); +x_70 = lean_ctor_get(x_4, 0); +lean_inc(x_70); +x_71 = lean_ctor_get(x_4, 1); +lean_inc(x_71); lean_dec(x_4); +x_72 = lean_box(x_5); lean_inc(x_1); -lean_inc(x_5); -lean_inc(x_53); -lean_inc(x_52); -lean_inc(x_51); -x_54 = lean_apply_5(x_1, x_51, x_52, x_53, x_5, x_6); -if (lean_obj_tag(x_54) == 0) +lean_inc(x_6); +lean_inc(x_71); +lean_inc(x_70); +lean_inc(x_69); +x_73 = lean_apply_6(x_1, x_69, x_70, x_71, x_72, x_6, x_7); +if (lean_obj_tag(x_73) == 0) { -lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_55 = lean_ctor_get(x_54, 1); -lean_inc(x_55); -lean_dec(x_54); -lean_inc(x_51); -x_56 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_56, 0, x_51); -x_57 = l_Lean_Elab_Info_updateContext_x3f(x_56, x_52); -x_58 = l_Lean_PersistentArray_toList___rarg(x_53); -x_59 = lean_box(0); -lean_inc(x_5); -lean_inc(x_2); -x_60 = l_List_mapM_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__20(x_1, x_2, x_57, x_58, x_59, x_5, x_55); -if (lean_obj_tag(x_60) == 0) +lean_object* x_74; uint8_t x_75; +x_74 = lean_ctor_get(x_73, 0); +lean_inc(x_74); +x_75 = lean_unbox(x_74); +lean_dec(x_74); +if (x_75 == 0) { -lean_object* x_61; lean_object* x_62; lean_object* x_63; -x_61 = lean_ctor_get(x_60, 0); -lean_inc(x_61); -x_62 = lean_ctor_get(x_60, 1); -lean_inc(x_62); -lean_dec(x_60); -x_63 = lean_apply_6(x_2, x_51, x_52, x_53, x_61, x_5, x_62); -if (lean_obj_tag(x_63) == 0) +lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; +lean_dec(x_1); +x_76 = lean_ctor_get(x_73, 1); +lean_inc(x_76); +lean_dec(x_73); +x_77 = lean_box(0); +x_78 = lean_box(x_5); +x_79 = lean_apply_7(x_2, x_69, x_70, x_71, x_77, x_78, x_6, x_76); +if (lean_obj_tag(x_79) == 0) { -lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_64 = lean_ctor_get(x_63, 0); -lean_inc(x_64); -x_65 = lean_ctor_get(x_63, 1); -lean_inc(x_65); -if (lean_is_exclusive(x_63)) { - lean_ctor_release(x_63, 0); - lean_ctor_release(x_63, 1); - x_66 = x_63; +lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; +x_80 = lean_ctor_get(x_79, 0); +lean_inc(x_80); +x_81 = lean_ctor_get(x_79, 1); +lean_inc(x_81); +if (lean_is_exclusive(x_79)) { + lean_ctor_release(x_79, 0); + lean_ctor_release(x_79, 1); + x_82 = x_79; } else { - lean_dec_ref(x_63); - x_66 = lean_box(0); + lean_dec_ref(x_79); + x_82 = lean_box(0); } -x_67 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_67, 0, x_64); -if (lean_is_scalar(x_66)) { - x_68 = lean_alloc_ctor(0, 2, 0); +x_83 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_83, 0, x_80); +if (lean_is_scalar(x_82)) { + x_84 = lean_alloc_ctor(0, 2, 0); } else { - x_68 = x_66; + x_84 = x_82; +} +lean_ctor_set(x_84, 0, x_83); +lean_ctor_set(x_84, 1, x_81); +return x_84; +} +else +{ +lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; +x_85 = lean_ctor_get(x_79, 0); +lean_inc(x_85); +x_86 = lean_ctor_get(x_79, 1); +lean_inc(x_86); +if (lean_is_exclusive(x_79)) { + lean_ctor_release(x_79, 0); + lean_ctor_release(x_79, 1); + x_87 = x_79; +} else { + lean_dec_ref(x_79); + x_87 = lean_box(0); +} +if (lean_is_scalar(x_87)) { + x_88 = lean_alloc_ctor(1, 2, 0); +} else { + x_88 = x_87; +} +lean_ctor_set(x_88, 0, x_85); +lean_ctor_set(x_88, 1, x_86); +return x_88; } -lean_ctor_set(x_68, 0, x_67); -lean_ctor_set(x_68, 1, x_65); -return x_68; } else { -lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; -x_69 = lean_ctor_get(x_63, 0); +lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; +x_89 = lean_ctor_get(x_73, 1); +lean_inc(x_89); +lean_dec(x_73); lean_inc(x_69); -x_70 = lean_ctor_get(x_63, 1); -lean_inc(x_70); -if (lean_is_exclusive(x_63)) { - lean_ctor_release(x_63, 0); - lean_ctor_release(x_63, 1); - x_71 = x_63; +x_90 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_90, 0, x_69); +x_91 = l_Lean_Elab_Info_updateContext_x3f(x_90, x_70); +x_92 = l_Lean_PersistentArray_toList___rarg(x_71); +x_93 = lean_box(0); +lean_inc(x_6); +lean_inc(x_2); +x_94 = l_List_mapM_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__23(x_1, x_2, x_91, x_92, x_93, x_5, x_6, x_89); +if (lean_obj_tag(x_94) == 0) +{ +lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; +x_95 = lean_ctor_get(x_94, 0); +lean_inc(x_95); +x_96 = lean_ctor_get(x_94, 1); +lean_inc(x_96); +lean_dec(x_94); +x_97 = lean_box(x_5); +x_98 = lean_apply_7(x_2, x_69, x_70, x_71, x_95, x_97, x_6, x_96); +if (lean_obj_tag(x_98) == 0) +{ +lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; +x_99 = lean_ctor_get(x_98, 0); +lean_inc(x_99); +x_100 = lean_ctor_get(x_98, 1); +lean_inc(x_100); +if (lean_is_exclusive(x_98)) { + lean_ctor_release(x_98, 0); + lean_ctor_release(x_98, 1); + x_101 = x_98; +} else { + lean_dec_ref(x_98); + x_101 = lean_box(0); +} +x_102 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_102, 0, x_99); +if (lean_is_scalar(x_101)) { + x_103 = lean_alloc_ctor(0, 2, 0); +} else { + x_103 = x_101; +} +lean_ctor_set(x_103, 0, x_102); +lean_ctor_set(x_103, 1, x_100); +return x_103; +} +else +{ +lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; +x_104 = lean_ctor_get(x_98, 0); +lean_inc(x_104); +x_105 = lean_ctor_get(x_98, 1); +lean_inc(x_105); +if (lean_is_exclusive(x_98)) { + lean_ctor_release(x_98, 0); + lean_ctor_release(x_98, 1); + x_106 = x_98; } else { - lean_dec_ref(x_63); - x_71 = lean_box(0); + lean_dec_ref(x_98); + x_106 = lean_box(0); } -if (lean_is_scalar(x_71)) { - x_72 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_106)) { + x_107 = lean_alloc_ctor(1, 2, 0); } else { - x_72 = x_71; + x_107 = x_106; } -lean_ctor_set(x_72, 0, x_69); -lean_ctor_set(x_72, 1, x_70); -return x_72; +lean_ctor_set(x_107, 0, x_104); +lean_ctor_set(x_107, 1, x_105); +return x_107; } } else { -lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; -lean_dec(x_53); -lean_dec(x_52); -lean_dec(x_51); -lean_dec(x_5); +lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; +lean_dec(x_71); +lean_dec(x_70); +lean_dec(x_69); +lean_dec(x_6); lean_dec(x_2); -x_73 = lean_ctor_get(x_60, 0); -lean_inc(x_73); -x_74 = lean_ctor_get(x_60, 1); -lean_inc(x_74); -if (lean_is_exclusive(x_60)) { - lean_ctor_release(x_60, 0); - lean_ctor_release(x_60, 1); - x_75 = x_60; +x_108 = lean_ctor_get(x_94, 0); +lean_inc(x_108); +x_109 = lean_ctor_get(x_94, 1); +lean_inc(x_109); +if (lean_is_exclusive(x_94)) { + lean_ctor_release(x_94, 0); + lean_ctor_release(x_94, 1); + x_110 = x_94; } else { - lean_dec_ref(x_60); - x_75 = lean_box(0); + lean_dec_ref(x_94); + x_110 = lean_box(0); } -if (lean_is_scalar(x_75)) { - x_76 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_110)) { + x_111 = lean_alloc_ctor(1, 2, 0); } else { - x_76 = x_75; + x_111 = x_110; +} +lean_ctor_set(x_111, 0, x_108); +lean_ctor_set(x_111, 1, x_109); +return x_111; } -lean_ctor_set(x_76, 0, x_73); -lean_ctor_set(x_76, 1, x_74); -return x_76; } } else { -lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; -lean_dec(x_53); -lean_dec(x_52); -lean_dec(x_51); -lean_dec(x_5); +lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; +lean_dec(x_71); +lean_dec(x_70); +lean_dec(x_69); +lean_dec(x_6); lean_dec(x_2); lean_dec(x_1); -x_77 = lean_ctor_get(x_54, 0); -lean_inc(x_77); -x_78 = lean_ctor_get(x_54, 1); -lean_inc(x_78); -if (lean_is_exclusive(x_54)) { - lean_ctor_release(x_54, 0); - lean_ctor_release(x_54, 1); - x_79 = x_54; +x_112 = lean_ctor_get(x_73, 0); +lean_inc(x_112); +x_113 = lean_ctor_get(x_73, 1); +lean_inc(x_113); +if (lean_is_exclusive(x_73)) { + lean_ctor_release(x_73, 0); + lean_ctor_release(x_73, 1); + x_114 = x_73; } else { - lean_dec_ref(x_54); - x_79 = lean_box(0); + lean_dec_ref(x_73); + x_114 = lean_box(0); } -if (lean_is_scalar(x_79)) { - x_80 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_114)) { + x_115 = lean_alloc_ctor(1, 2, 0); } else { - x_80 = x_79; + x_115 = x_114; } -lean_ctor_set(x_80, 0, x_77); -lean_ctor_set(x_80, 1, x_78); -return x_80; +lean_ctor_set(x_115, 0, x_112); +lean_ctor_set(x_115, 1, x_113); +return x_115; } } } default: { -lean_object* x_81; lean_object* x_82; -lean_dec(x_5); +lean_object* x_116; lean_object* x_117; +lean_dec(x_6); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_81 = lean_box(0); -x_82 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_82, 0, x_81); -lean_ctor_set(x_82, 1, x_6); -return x_82; -} -} +x_116 = lean_box(0); +x_117 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_117, 0, x_116); +lean_ctor_set(x_117, 1, x_7); +return x_117; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_UnusedVariables_collectReferences___spec__17(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; lean_object* x_7; -x_6 = lean_box(0); -x_7 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18(x_1, x_2, x_6, x_3, x_4, x_5); -return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences___spec__16___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__20___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_8; -x_8 = lean_apply_5(x_1, x_2, x_3, x_4, x_6, x_7); -return x_8; +lean_object* x_9; lean_object* x_10; +x_9 = lean_box(x_6); +x_10 = lean_apply_6(x_1, x_2, x_3, x_4, x_9, x_7, x_8); +return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences___spec__16(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__20(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, lean_object* x_6, lean_object* x_7) { _start: { -lean_object* x_6; lean_object* x_7; -x_6 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences___spec__16___lambda__1___boxed), 7, 1); -lean_closure_set(x_6, 0, x_2); -x_7 = l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_UnusedVariables_collectReferences___spec__17(x_1, x_6, x_3, x_4, x_5); -if (lean_obj_tag(x_7) == 0) +lean_object* x_8; lean_object* x_9; +x_8 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__20___lambda__1___boxed), 8, 1); +lean_closure_set(x_8, 0, x_2); +x_9 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21(x_1, x_8, x_3, x_4, x_5, x_6, x_7); +if (lean_obj_tag(x_9) == 0) { -uint8_t x_8; -x_8 = !lean_is_exclusive(x_7); -if (x_8 == 0) +uint8_t x_10; +x_10 = !lean_is_exclusive(x_9); +if (x_10 == 0) { -lean_object* x_9; lean_object* x_10; -x_9 = lean_ctor_get(x_7, 0); -lean_dec(x_9); -x_10 = lean_box(0); -lean_ctor_set(x_7, 0, x_10); -return x_7; +lean_object* x_11; lean_object* x_12; +x_11 = lean_ctor_get(x_9, 0); +lean_dec(x_11); +x_12 = lean_box(0); +lean_ctor_set(x_9, 0, x_12); +return x_9; } else { -lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_11 = lean_ctor_get(x_7, 1); -lean_inc(x_11); -lean_dec(x_7); -x_12 = lean_box(0); -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_12); -lean_ctor_set(x_13, 1, x_11); -return x_13; +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_9, 1); +lean_inc(x_13); +lean_dec(x_9); +x_14 = lean_box(0); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_13); +return x_15; } } else { -uint8_t x_14; -x_14 = !lean_is_exclusive(x_7); -if (x_14 == 0) +uint8_t x_16; +x_16 = !lean_is_exclusive(x_9); +if (x_16 == 0) { -return x_7; +return x_9; } else { -lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = lean_ctor_get(x_7, 0); -x_16 = lean_ctor_get(x_7, 1); -lean_inc(x_16); -lean_inc(x_15); -lean_dec(x_7); -x_17 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_17, 0, x_15); -lean_ctor_set(x_17, 1, x_16); -return x_17; +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_9, 0); +x_18 = lean_ctor_get(x_9, 1); +lean_inc(x_18); +lean_inc(x_17); +lean_dec(x_9); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set(x_19, 1, x_18); +return x_19; } } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__1(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_9 = lean_st_ref_take(x_7, x_8); -x_10 = lean_ctor_get(x_9, 0); -lean_inc(x_10); -x_11 = lean_ctor_get(x_10, 1); -lean_inc(x_11); -x_12 = !lean_is_exclusive(x_9); -if (x_12 == 0) +lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; +x_6 = lean_st_ref_take(x_4, x_5); +x_7 = lean_ctor_get(x_6, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_6, 1); +lean_inc(x_8); +lean_dec(x_6); +x_9 = !lean_is_exclusive(x_7); +if (x_9 == 0) { -lean_object* x_13; lean_object* x_14; uint8_t x_15; -x_13 = lean_ctor_get(x_9, 1); -x_14 = lean_ctor_get(x_9, 0); -lean_dec(x_14); -x_15 = !lean_is_exclusive(x_11); +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_10 = lean_ctor_get(x_7, 4); +x_11 = lean_ctor_get(x_1, 3); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 7); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_array_push(x_10, x_12); +lean_ctor_set(x_7, 4, x_13); +x_14 = lean_st_ref_set(x_4, x_7, x_8); +x_15 = !lean_is_exclusive(x_14); if (x_15 == 0) { -lean_object* x_16; lean_object* x_17; lean_object* x_18; uint64_t x_19; uint64_t x_20; uint64_t x_21; uint64_t x_22; uint64_t x_23; uint64_t x_24; uint64_t x_25; size_t x_26; size_t x_27; size_t x_28; size_t x_29; size_t x_30; lean_object* x_31; lean_object* x_32; -x_16 = lean_ctor_get(x_11, 0); -x_17 = lean_ctor_get(x_11, 1); -x_18 = lean_array_get_size(x_17); -x_19 = l___private_Lean_Syntax_0__String_hashRange____x40_Lean_Syntax___hyg_169_(x_1); -x_20 = 32; -x_21 = lean_uint64_shift_right(x_19, x_20); -x_22 = lean_uint64_xor(x_19, x_21); -x_23 = 16; -x_24 = lean_uint64_shift_right(x_22, x_23); -x_25 = lean_uint64_xor(x_22, x_24); -x_26 = lean_uint64_to_usize(x_25); -x_27 = lean_usize_of_nat(x_18); -lean_dec(x_18); -x_28 = 1; -x_29 = lean_usize_sub(x_27, x_28); -x_30 = lean_usize_land(x_26, x_29); -x_31 = lean_array_uget(x_17, x_30); -x_32 = l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_collectReferences___spec__1(x_1, x_31); -if (lean_obj_tag(x_32) == 0) -{ -lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; -x_33 = lean_ctor_get(x_10, 0); -lean_inc(x_33); -x_34 = l_Lean_LocalDecl_userName(x_2); -x_35 = lean_box(0); -lean_ctor_set_tag(x_9, 1); -lean_ctor_set(x_9, 1, x_35); -lean_ctor_set(x_9, 0, x_3); -x_36 = lean_array_mk(x_9); -x_37 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_37, 0, x_34); -lean_ctor_set(x_37, 1, x_4); -lean_ctor_set(x_37, 2, x_5); -lean_ctor_set(x_37, 3, x_36); -x_38 = lean_ctor_get(x_10, 2); -lean_inc(x_38); -x_39 = lean_ctor_get(x_10, 3); -lean_inc(x_39); -x_40 = lean_ctor_get(x_10, 4); -lean_inc(x_40); -lean_dec(x_10); -x_41 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__2(x_1, x_31); -if (x_41 == 0) -{ -lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; uint8_t x_51; -x_42 = lean_unsigned_to_nat(1u); -x_43 = lean_nat_add(x_16, x_42); +lean_object* x_16; uint8_t x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_14, 0); lean_dec(x_16); -x_44 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_44, 0, x_1); -lean_ctor_set(x_44, 1, x_37); -lean_ctor_set(x_44, 2, x_31); -x_45 = lean_array_uset(x_17, x_30, x_44); -x_46 = lean_unsigned_to_nat(4u); -x_47 = lean_nat_mul(x_43, x_46); -x_48 = lean_unsigned_to_nat(3u); -x_49 = lean_nat_div(x_47, x_48); -lean_dec(x_47); -x_50 = lean_array_get_size(x_45); -x_51 = lean_nat_dec_le(x_49, x_50); -lean_dec(x_50); -lean_dec(x_49); -if (x_51 == 0) -{ -lean_object* x_52; lean_object* x_53; lean_object* x_54; uint8_t x_55; -x_52 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__3(x_45); -lean_ctor_set(x_11, 1, x_52); -lean_ctor_set(x_11, 0, x_43); -x_53 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_53, 0, x_33); -lean_ctor_set(x_53, 1, x_11); -lean_ctor_set(x_53, 2, x_38); -lean_ctor_set(x_53, 3, x_39); -lean_ctor_set(x_53, 4, x_40); -x_54 = lean_st_ref_set(x_7, x_53, x_13); -x_55 = !lean_is_exclusive(x_54); -if (x_55 == 0) -{ -lean_object* x_56; lean_object* x_57; -x_56 = lean_ctor_get(x_54, 0); -lean_dec(x_56); -x_57 = lean_box(0); -lean_ctor_set(x_54, 0, x_57); -return x_54; +x_17 = 1; +x_18 = lean_box(x_17); +lean_ctor_set(x_14, 0, x_18); +return x_14; } else { -lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_58 = lean_ctor_get(x_54, 1); -lean_inc(x_58); -lean_dec(x_54); -x_59 = lean_box(0); -x_60 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_60, 0, x_59); -lean_ctor_set(x_60, 1, x_58); -return x_60; +lean_object* x_19; uint8_t x_20; lean_object* x_21; lean_object* x_22; +x_19 = lean_ctor_get(x_14, 1); +lean_inc(x_19); +lean_dec(x_14); +x_20 = 1; +x_21 = lean_box(x_20); +x_22 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_22, 0, x_21); +lean_ctor_set(x_22, 1, x_19); +return x_22; } } else { -lean_object* x_61; lean_object* x_62; uint8_t x_63; -lean_ctor_set(x_11, 1, x_45); -lean_ctor_set(x_11, 0, x_43); -x_61 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_61, 0, x_33); -lean_ctor_set(x_61, 1, x_11); -lean_ctor_set(x_61, 2, x_38); -lean_ctor_set(x_61, 3, x_39); -lean_ctor_set(x_61, 4, x_40); -x_62 = lean_st_ref_set(x_7, x_61, x_13); -x_63 = !lean_is_exclusive(x_62); -if (x_63 == 0) -{ -lean_object* x_64; lean_object* x_65; -x_64 = lean_ctor_get(x_62, 0); -lean_dec(x_64); -x_65 = lean_box(0); -lean_ctor_set(x_62, 0, x_65); -return x_62; -} +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; lean_object* x_36; lean_object* x_37; +x_23 = lean_ctor_get(x_7, 0); +x_24 = lean_ctor_get(x_7, 1); +x_25 = lean_ctor_get(x_7, 2); +x_26 = lean_ctor_get(x_7, 3); +x_27 = lean_ctor_get(x_7, 4); +lean_inc(x_27); +lean_inc(x_26); +lean_inc(x_25); +lean_inc(x_24); +lean_inc(x_23); +lean_dec(x_7); +x_28 = lean_ctor_get(x_1, 3); +lean_inc(x_28); +lean_dec(x_1); +x_29 = lean_ctor_get(x_28, 7); +lean_inc(x_29); +lean_dec(x_28); +x_30 = lean_array_push(x_27, x_29); +x_31 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_31, 0, x_23); +lean_ctor_set(x_31, 1, x_24); +lean_ctor_set(x_31, 2, x_25); +lean_ctor_set(x_31, 3, x_26); +lean_ctor_set(x_31, 4, x_30); +x_32 = lean_st_ref_set(x_4, x_31, x_8); +x_33 = lean_ctor_get(x_32, 1); +lean_inc(x_33); +if (lean_is_exclusive(x_32)) { + lean_ctor_release(x_32, 0); + lean_ctor_release(x_32, 1); + x_34 = x_32; +} else { + lean_dec_ref(x_32); + x_34 = lean_box(0); +} +x_35 = 1; +x_36 = lean_box(x_35); +if (lean_is_scalar(x_34)) { + x_37 = lean_alloc_ctor(0, 2, 0); +} else { + x_37 = x_34; +} +lean_ctor_set(x_37, 0, x_36); +lean_ctor_set(x_37, 1, x_33); +return x_37; +} +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__2(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; lean_object* x_6; lean_object* x_7; +x_5 = 1; +x_6 = lean_box(x_5); +x_7 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_7, 0, x_6); +lean_ctor_set(x_7, 1, x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, uint8_t x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; +x_17 = lean_st_ref_take(x_9, x_10); +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_18, 1); +lean_inc(x_19); +x_20 = !lean_is_exclusive(x_17); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_21 = lean_ctor_get(x_17, 1); +x_22 = lean_ctor_get(x_17, 0); +lean_dec(x_22); +x_23 = !lean_is_exclusive(x_19); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; uint64_t x_27; uint64_t x_28; uint64_t x_29; uint64_t x_30; uint64_t x_31; uint64_t x_32; uint64_t x_33; size_t x_34; size_t x_35; size_t x_36; size_t x_37; size_t x_38; lean_object* x_39; lean_object* x_40; +x_24 = lean_ctor_get(x_19, 0); +x_25 = lean_ctor_get(x_19, 1); +x_26 = lean_array_get_size(x_25); +x_27 = l___private_Lean_Syntax_0__String_hashRange____x40_Lean_Syntax___hyg_169_(x_2); +x_28 = 32; +x_29 = lean_uint64_shift_right(x_27, x_28); +x_30 = lean_uint64_xor(x_27, x_29); +x_31 = 16; +x_32 = lean_uint64_shift_right(x_30, x_31); +x_33 = lean_uint64_xor(x_30, x_32); +x_34 = lean_uint64_to_usize(x_33); +x_35 = lean_usize_of_nat(x_26); +lean_dec(x_26); +x_36 = 1; +x_37 = lean_usize_sub(x_35, x_36); +x_38 = lean_usize_land(x_34, x_37); +x_39 = lean_array_uget(x_25, x_38); +x_40 = l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__1(x_2, x_39); +if (lean_obj_tag(x_40) == 0) +{ +lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; +x_41 = lean_ctor_get(x_18, 0); +lean_inc(x_41); +x_42 = l_Lean_LocalDecl_userName(x_3); +x_43 = lean_box(0); +lean_ctor_set_tag(x_17, 1); +lean_ctor_set(x_17, 1, x_43); +lean_ctor_set(x_17, 0, x_4); +x_44 = lean_array_mk(x_17); +x_45 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_45, 0, x_42); +lean_ctor_set(x_45, 1, x_5); +lean_ctor_set(x_45, 2, x_6); +lean_ctor_set(x_45, 3, x_44); +x_46 = lean_ctor_get(x_18, 2); +lean_inc(x_46); +x_47 = lean_ctor_get(x_18, 3); +lean_inc(x_47); +x_48 = lean_ctor_get(x_18, 4); +lean_inc(x_48); +lean_dec(x_18); +x_49 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__2(x_2, x_39); +if (x_49 == 0) +{ +lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; uint8_t x_59; +x_50 = lean_unsigned_to_nat(1u); +x_51 = lean_nat_add(x_24, x_50); +lean_dec(x_24); +x_52 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_52, 0, x_2); +lean_ctor_set(x_52, 1, x_45); +lean_ctor_set(x_52, 2, x_39); +x_53 = lean_array_uset(x_25, x_38, x_52); +x_54 = lean_unsigned_to_nat(4u); +x_55 = lean_nat_mul(x_51, x_54); +x_56 = lean_unsigned_to_nat(3u); +x_57 = lean_nat_div(x_55, x_56); +lean_dec(x_55); +x_58 = lean_array_get_size(x_53); +x_59 = lean_nat_dec_le(x_57, x_58); +lean_dec(x_58); +lean_dec(x_57); +if (x_59 == 0) +{ +lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; +x_60 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__3(x_53); +lean_ctor_set(x_19, 1, x_60); +lean_ctor_set(x_19, 0, x_51); +x_61 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_61, 0, x_41); +lean_ctor_set(x_61, 1, x_19); +lean_ctor_set(x_61, 2, x_46); +lean_ctor_set(x_61, 3, x_47); +lean_ctor_set(x_61, 4, x_48); +x_62 = lean_st_ref_set(x_9, x_61, x_21); +x_63 = !lean_is_exclusive(x_62); +if (x_63 == 0) +{ +lean_object* x_64; lean_object* x_65; +x_64 = lean_ctor_get(x_62, 0); +lean_dec(x_64); +x_65 = lean_box(0); +lean_ctor_set(x_62, 0, x_65); +x_11 = x_62; +goto block_16; +} else { lean_object* x_66; lean_object* x_67; lean_object* x_68; @@ -10792,151 +11323,156 @@ x_67 = lean_box(0); x_68 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_68, 0, x_67); lean_ctor_set(x_68, 1, x_66); -return x_68; -} +x_11 = x_68; +goto block_16; } } else { -lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; uint8_t x_75; -x_69 = lean_box(0); -x_70 = lean_array_uset(x_17, x_30, x_69); -x_71 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__6(x_1, x_37, x_31); -x_72 = lean_array_uset(x_70, x_30, x_71); -lean_ctor_set(x_11, 1, x_72); -x_73 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_73, 0, x_33); -lean_ctor_set(x_73, 1, x_11); -lean_ctor_set(x_73, 2, x_38); -lean_ctor_set(x_73, 3, x_39); -lean_ctor_set(x_73, 4, x_40); -x_74 = lean_st_ref_set(x_7, x_73, x_13); -x_75 = !lean_is_exclusive(x_74); -if (x_75 == 0) +lean_object* x_69; lean_object* x_70; uint8_t x_71; +lean_ctor_set(x_19, 1, x_53); +lean_ctor_set(x_19, 0, x_51); +x_69 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_69, 0, x_41); +lean_ctor_set(x_69, 1, x_19); +lean_ctor_set(x_69, 2, x_46); +lean_ctor_set(x_69, 3, x_47); +lean_ctor_set(x_69, 4, x_48); +x_70 = lean_st_ref_set(x_9, x_69, x_21); +x_71 = !lean_is_exclusive(x_70); +if (x_71 == 0) { -lean_object* x_76; lean_object* x_77; -x_76 = lean_ctor_get(x_74, 0); -lean_dec(x_76); -x_77 = lean_box(0); -lean_ctor_set(x_74, 0, x_77); -return x_74; +lean_object* x_72; lean_object* x_73; +x_72 = lean_ctor_get(x_70, 0); +lean_dec(x_72); +x_73 = lean_box(0); +lean_ctor_set(x_70, 0, x_73); +x_11 = x_70; +goto block_16; } else { -lean_object* x_78; lean_object* x_79; lean_object* x_80; -x_78 = lean_ctor_get(x_74, 1); -lean_inc(x_78); -lean_dec(x_74); -x_79 = lean_box(0); -x_80 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_80, 0, x_79); -lean_ctor_set(x_80, 1, x_78); -return x_80; +lean_object* x_74; lean_object* x_75; lean_object* x_76; +x_74 = lean_ctor_get(x_70, 1); +lean_inc(x_74); +lean_dec(x_70); +x_75 = lean_box(0); +x_76 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_76, 0, x_75); +lean_ctor_set(x_76, 1, x_74); +x_11 = x_76; +goto block_16; } } } else { -lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; uint8_t x_92; -lean_free_object(x_9); -lean_dec(x_5); -lean_dec(x_4); -x_81 = lean_ctor_get(x_32, 0); -lean_inc(x_81); -lean_dec(x_32); -x_82 = lean_ctor_get(x_10, 0); -lean_inc(x_82); -x_83 = lean_ctor_get(x_81, 0); -lean_inc(x_83); -x_84 = lean_ctor_get(x_81, 1); -lean_inc(x_84); -x_85 = lean_ctor_get(x_81, 2); -lean_inc(x_85); -x_86 = lean_ctor_get(x_81, 3); -lean_inc(x_86); -lean_dec(x_81); -x_87 = lean_array_push(x_86, x_3); -x_88 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_88, 0, x_83); -lean_ctor_set(x_88, 1, x_84); -lean_ctor_set(x_88, 2, x_85); -lean_ctor_set(x_88, 3, x_87); -x_89 = lean_ctor_get(x_10, 2); -lean_inc(x_89); -x_90 = lean_ctor_get(x_10, 3); -lean_inc(x_90); -x_91 = lean_ctor_get(x_10, 4); -lean_inc(x_91); -lean_dec(x_10); -x_92 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__2(x_1, x_31); -if (x_92 == 0) -{ -lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; uint8_t x_102; -x_93 = lean_unsigned_to_nat(1u); -x_94 = lean_nat_add(x_16, x_93); -lean_dec(x_16); -x_95 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_95, 0, x_1); -lean_ctor_set(x_95, 1, x_88); -lean_ctor_set(x_95, 2, x_31); -x_96 = lean_array_uset(x_17, x_30, x_95); -x_97 = lean_unsigned_to_nat(4u); -x_98 = lean_nat_mul(x_94, x_97); -x_99 = lean_unsigned_to_nat(3u); -x_100 = lean_nat_div(x_98, x_99); -lean_dec(x_98); -x_101 = lean_array_get_size(x_96); -x_102 = lean_nat_dec_le(x_100, x_101); -lean_dec(x_101); -lean_dec(x_100); -if (x_102 == 0) +lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; uint8_t x_83; +x_77 = lean_box(0); +x_78 = lean_array_uset(x_25, x_38, x_77); +x_79 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__6(x_2, x_45, x_39); +x_80 = lean_array_uset(x_78, x_38, x_79); +lean_ctor_set(x_19, 1, x_80); +x_81 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_81, 0, x_41); +lean_ctor_set(x_81, 1, x_19); +lean_ctor_set(x_81, 2, x_46); +lean_ctor_set(x_81, 3, x_47); +lean_ctor_set(x_81, 4, x_48); +x_82 = lean_st_ref_set(x_9, x_81, x_21); +x_83 = !lean_is_exclusive(x_82); +if (x_83 == 0) { -lean_object* x_103; lean_object* x_104; lean_object* x_105; uint8_t x_106; -x_103 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__3(x_96); -lean_ctor_set(x_11, 1, x_103); -lean_ctor_set(x_11, 0, x_94); -x_104 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_104, 0, x_82); -lean_ctor_set(x_104, 1, x_11); -lean_ctor_set(x_104, 2, x_89); -lean_ctor_set(x_104, 3, x_90); -lean_ctor_set(x_104, 4, x_91); -x_105 = lean_st_ref_set(x_7, x_104, x_13); -x_106 = !lean_is_exclusive(x_105); -if (x_106 == 0) -{ -lean_object* x_107; lean_object* x_108; -x_107 = lean_ctor_get(x_105, 0); -lean_dec(x_107); -x_108 = lean_box(0); -lean_ctor_set(x_105, 0, x_108); -return x_105; +lean_object* x_84; lean_object* x_85; +x_84 = lean_ctor_get(x_82, 0); +lean_dec(x_84); +x_85 = lean_box(0); +lean_ctor_set(x_82, 0, x_85); +x_11 = x_82; +goto block_16; } else { -lean_object* x_109; lean_object* x_110; lean_object* x_111; -x_109 = lean_ctor_get(x_105, 1); -lean_inc(x_109); -lean_dec(x_105); -x_110 = lean_box(0); -x_111 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_111, 0, x_110); -lean_ctor_set(x_111, 1, x_109); -return x_111; +lean_object* x_86; lean_object* x_87; lean_object* x_88; +x_86 = lean_ctor_get(x_82, 1); +lean_inc(x_86); +lean_dec(x_82); +x_87 = lean_box(0); +x_88 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_88, 0, x_87); +lean_ctor_set(x_88, 1, x_86); +x_11 = x_88; +goto block_16; +} } } else { -lean_object* x_112; lean_object* x_113; uint8_t x_114; -lean_ctor_set(x_11, 1, x_96); -lean_ctor_set(x_11, 0, x_94); +lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; uint8_t x_100; +lean_free_object(x_17); +lean_dec(x_6); +lean_dec(x_5); +x_89 = lean_ctor_get(x_40, 0); +lean_inc(x_89); +lean_dec(x_40); +x_90 = lean_ctor_get(x_18, 0); +lean_inc(x_90); +x_91 = lean_ctor_get(x_89, 0); +lean_inc(x_91); +x_92 = lean_ctor_get(x_89, 1); +lean_inc(x_92); +x_93 = lean_ctor_get(x_89, 2); +lean_inc(x_93); +x_94 = lean_ctor_get(x_89, 3); +lean_inc(x_94); +lean_dec(x_89); +x_95 = lean_array_push(x_94, x_4); +x_96 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_96, 0, x_91); +lean_ctor_set(x_96, 1, x_92); +lean_ctor_set(x_96, 2, x_93); +lean_ctor_set(x_96, 3, x_95); +x_97 = lean_ctor_get(x_18, 2); +lean_inc(x_97); +x_98 = lean_ctor_get(x_18, 3); +lean_inc(x_98); +x_99 = lean_ctor_get(x_18, 4); +lean_inc(x_99); +lean_dec(x_18); +x_100 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__2(x_2, x_39); +if (x_100 == 0) +{ +lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; uint8_t x_110; +x_101 = lean_unsigned_to_nat(1u); +x_102 = lean_nat_add(x_24, x_101); +lean_dec(x_24); +x_103 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_103, 0, x_2); +lean_ctor_set(x_103, 1, x_96); +lean_ctor_set(x_103, 2, x_39); +x_104 = lean_array_uset(x_25, x_38, x_103); +x_105 = lean_unsigned_to_nat(4u); +x_106 = lean_nat_mul(x_102, x_105); +x_107 = lean_unsigned_to_nat(3u); +x_108 = lean_nat_div(x_106, x_107); +lean_dec(x_106); +x_109 = lean_array_get_size(x_104); +x_110 = lean_nat_dec_le(x_108, x_109); +lean_dec(x_109); +lean_dec(x_108); +if (x_110 == 0) +{ +lean_object* x_111; lean_object* x_112; lean_object* x_113; uint8_t x_114; +x_111 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__3(x_104); +lean_ctor_set(x_19, 1, x_111); +lean_ctor_set(x_19, 0, x_102); x_112 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_112, 0, x_82); -lean_ctor_set(x_112, 1, x_11); -lean_ctor_set(x_112, 2, x_89); -lean_ctor_set(x_112, 3, x_90); -lean_ctor_set(x_112, 4, x_91); -x_113 = lean_st_ref_set(x_7, x_112, x_13); +lean_ctor_set(x_112, 0, x_90); +lean_ctor_set(x_112, 1, x_19); +lean_ctor_set(x_112, 2, x_97); +lean_ctor_set(x_112, 3, x_98); +lean_ctor_set(x_112, 4, x_99); +x_113 = lean_st_ref_set(x_9, x_112, x_21); x_114 = !lean_is_exclusive(x_113); if (x_114 == 0) { @@ -10945,7 +11481,8 @@ x_115 = lean_ctor_get(x_113, 0); lean_dec(x_115); x_116 = lean_box(0); lean_ctor_set(x_113, 0, x_116); -return x_113; +x_11 = x_113; +goto block_16; } else { @@ -10957,757 +11494,821 @@ x_118 = lean_box(0); x_119 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_119, 0, x_118); lean_ctor_set(x_119, 1, x_117); -return x_119; -} +x_11 = x_119; +goto block_16; } } else { -lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; uint8_t x_126; -x_120 = lean_box(0); -x_121 = lean_array_uset(x_17, x_30, x_120); -x_122 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__6(x_1, x_88, x_31); -x_123 = lean_array_uset(x_121, x_30, x_122); -lean_ctor_set(x_11, 1, x_123); -x_124 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_124, 0, x_82); -lean_ctor_set(x_124, 1, x_11); -lean_ctor_set(x_124, 2, x_89); -lean_ctor_set(x_124, 3, x_90); -lean_ctor_set(x_124, 4, x_91); -x_125 = lean_st_ref_set(x_7, x_124, x_13); -x_126 = !lean_is_exclusive(x_125); -if (x_126 == 0) -{ -lean_object* x_127; lean_object* x_128; -x_127 = lean_ctor_get(x_125, 0); -lean_dec(x_127); -x_128 = lean_box(0); -lean_ctor_set(x_125, 0, x_128); -return x_125; +lean_object* x_120; lean_object* x_121; uint8_t x_122; +lean_ctor_set(x_19, 1, x_104); +lean_ctor_set(x_19, 0, x_102); +x_120 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_120, 0, x_90); +lean_ctor_set(x_120, 1, x_19); +lean_ctor_set(x_120, 2, x_97); +lean_ctor_set(x_120, 3, x_98); +lean_ctor_set(x_120, 4, x_99); +x_121 = lean_st_ref_set(x_9, x_120, x_21); +x_122 = !lean_is_exclusive(x_121); +if (x_122 == 0) +{ +lean_object* x_123; lean_object* x_124; +x_123 = lean_ctor_get(x_121, 0); +lean_dec(x_123); +x_124 = lean_box(0); +lean_ctor_set(x_121, 0, x_124); +x_11 = x_121; +goto block_16; } else { -lean_object* x_129; lean_object* x_130; lean_object* x_131; -x_129 = lean_ctor_get(x_125, 1); -lean_inc(x_129); -lean_dec(x_125); -x_130 = lean_box(0); -x_131 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_131, 0, x_130); -lean_ctor_set(x_131, 1, x_129); -return x_131; -} +lean_object* x_125; lean_object* x_126; lean_object* x_127; +x_125 = lean_ctor_get(x_121, 1); +lean_inc(x_125); +lean_dec(x_121); +x_126 = lean_box(0); +x_127 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_127, 0, x_126); +lean_ctor_set(x_127, 1, x_125); +x_11 = x_127; +goto block_16; } } } else { -lean_object* x_132; lean_object* x_133; lean_object* x_134; uint64_t x_135; uint64_t x_136; uint64_t x_137; uint64_t x_138; uint64_t x_139; uint64_t x_140; uint64_t x_141; size_t x_142; size_t x_143; size_t x_144; size_t x_145; size_t x_146; lean_object* x_147; lean_object* x_148; -x_132 = lean_ctor_get(x_11, 0); -x_133 = lean_ctor_get(x_11, 1); -lean_inc(x_133); -lean_inc(x_132); -lean_dec(x_11); -x_134 = lean_array_get_size(x_133); -x_135 = l___private_Lean_Syntax_0__String_hashRange____x40_Lean_Syntax___hyg_169_(x_1); -x_136 = 32; -x_137 = lean_uint64_shift_right(x_135, x_136); -x_138 = lean_uint64_xor(x_135, x_137); -x_139 = 16; -x_140 = lean_uint64_shift_right(x_138, x_139); -x_141 = lean_uint64_xor(x_138, x_140); -x_142 = lean_uint64_to_usize(x_141); -x_143 = lean_usize_of_nat(x_134); -lean_dec(x_134); -x_144 = 1; -x_145 = lean_usize_sub(x_143, x_144); -x_146 = lean_usize_land(x_142, x_145); -x_147 = lean_array_uget(x_133, x_146); -x_148 = l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_collectReferences___spec__1(x_1, x_147); -if (lean_obj_tag(x_148) == 0) -{ -lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; uint8_t x_157; -x_149 = lean_ctor_get(x_10, 0); -lean_inc(x_149); -x_150 = l_Lean_LocalDecl_userName(x_2); -x_151 = lean_box(0); -lean_ctor_set_tag(x_9, 1); -lean_ctor_set(x_9, 1, x_151); -lean_ctor_set(x_9, 0, x_3); -x_152 = lean_array_mk(x_9); -x_153 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_153, 0, x_150); -lean_ctor_set(x_153, 1, x_4); -lean_ctor_set(x_153, 2, x_5); -lean_ctor_set(x_153, 3, x_152); -x_154 = lean_ctor_get(x_10, 2); -lean_inc(x_154); -x_155 = lean_ctor_get(x_10, 3); -lean_inc(x_155); -x_156 = lean_ctor_get(x_10, 4); -lean_inc(x_156); -lean_dec(x_10); -x_157 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__2(x_1, x_147); -if (x_157 == 0) -{ -lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; uint8_t x_167; -x_158 = lean_unsigned_to_nat(1u); -x_159 = lean_nat_add(x_132, x_158); -lean_dec(x_132); -x_160 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_160, 0, x_1); -lean_ctor_set(x_160, 1, x_153); -lean_ctor_set(x_160, 2, x_147); -x_161 = lean_array_uset(x_133, x_146, x_160); -x_162 = lean_unsigned_to_nat(4u); -x_163 = lean_nat_mul(x_159, x_162); -x_164 = lean_unsigned_to_nat(3u); -x_165 = lean_nat_div(x_163, x_164); -lean_dec(x_163); -x_166 = lean_array_get_size(x_161); -x_167 = lean_nat_dec_le(x_165, x_166); -lean_dec(x_166); -lean_dec(x_165); -if (x_167 == 0) +lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; uint8_t x_134; +x_128 = lean_box(0); +x_129 = lean_array_uset(x_25, x_38, x_128); +x_130 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__6(x_2, x_96, x_39); +x_131 = lean_array_uset(x_129, x_38, x_130); +lean_ctor_set(x_19, 1, x_131); +x_132 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_132, 0, x_90); +lean_ctor_set(x_132, 1, x_19); +lean_ctor_set(x_132, 2, x_97); +lean_ctor_set(x_132, 3, x_98); +lean_ctor_set(x_132, 4, x_99); +x_133 = lean_st_ref_set(x_9, x_132, x_21); +x_134 = !lean_is_exclusive(x_133); +if (x_134 == 0) { -lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; -x_168 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__3(x_161); -x_169 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_169, 0, x_159); -lean_ctor_set(x_169, 1, x_168); -x_170 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_170, 0, x_149); -lean_ctor_set(x_170, 1, x_169); -lean_ctor_set(x_170, 2, x_154); -lean_ctor_set(x_170, 3, x_155); -lean_ctor_set(x_170, 4, x_156); -x_171 = lean_st_ref_set(x_7, x_170, x_13); -x_172 = lean_ctor_get(x_171, 1); -lean_inc(x_172); -if (lean_is_exclusive(x_171)) { - lean_ctor_release(x_171, 0); - lean_ctor_release(x_171, 1); - x_173 = x_171; -} else { - lean_dec_ref(x_171); - x_173 = lean_box(0); +lean_object* x_135; lean_object* x_136; +x_135 = lean_ctor_get(x_133, 0); +lean_dec(x_135); +x_136 = lean_box(0); +lean_ctor_set(x_133, 0, x_136); +x_11 = x_133; +goto block_16; +} +else +{ +lean_object* x_137; lean_object* x_138; lean_object* x_139; +x_137 = lean_ctor_get(x_133, 1); +lean_inc(x_137); +lean_dec(x_133); +x_138 = lean_box(0); +x_139 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_139, 0, x_138); +lean_ctor_set(x_139, 1, x_137); +x_11 = x_139; +goto block_16; +} } -x_174 = lean_box(0); -if (lean_is_scalar(x_173)) { - x_175 = lean_alloc_ctor(0, 2, 0); -} else { - x_175 = x_173; } -lean_ctor_set(x_175, 0, x_174); -lean_ctor_set(x_175, 1, x_172); -return x_175; } else { -lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; -x_176 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_176, 0, x_159); -lean_ctor_set(x_176, 1, x_161); -x_177 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_177, 0, x_149); +lean_object* x_140; lean_object* x_141; lean_object* x_142; uint64_t x_143; uint64_t x_144; uint64_t x_145; uint64_t x_146; uint64_t x_147; uint64_t x_148; uint64_t x_149; size_t x_150; size_t x_151; size_t x_152; size_t x_153; size_t x_154; lean_object* x_155; lean_object* x_156; +x_140 = lean_ctor_get(x_19, 0); +x_141 = lean_ctor_get(x_19, 1); +lean_inc(x_141); +lean_inc(x_140); +lean_dec(x_19); +x_142 = lean_array_get_size(x_141); +x_143 = l___private_Lean_Syntax_0__String_hashRange____x40_Lean_Syntax___hyg_169_(x_2); +x_144 = 32; +x_145 = lean_uint64_shift_right(x_143, x_144); +x_146 = lean_uint64_xor(x_143, x_145); +x_147 = 16; +x_148 = lean_uint64_shift_right(x_146, x_147); +x_149 = lean_uint64_xor(x_146, x_148); +x_150 = lean_uint64_to_usize(x_149); +x_151 = lean_usize_of_nat(x_142); +lean_dec(x_142); +x_152 = 1; +x_153 = lean_usize_sub(x_151, x_152); +x_154 = lean_usize_land(x_150, x_153); +x_155 = lean_array_uget(x_141, x_154); +x_156 = l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__1(x_2, x_155); +if (lean_obj_tag(x_156) == 0) +{ +lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; uint8_t x_165; +x_157 = lean_ctor_get(x_18, 0); +lean_inc(x_157); +x_158 = l_Lean_LocalDecl_userName(x_3); +x_159 = lean_box(0); +lean_ctor_set_tag(x_17, 1); +lean_ctor_set(x_17, 1, x_159); +lean_ctor_set(x_17, 0, x_4); +x_160 = lean_array_mk(x_17); +x_161 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_161, 0, x_158); +lean_ctor_set(x_161, 1, x_5); +lean_ctor_set(x_161, 2, x_6); +lean_ctor_set(x_161, 3, x_160); +x_162 = lean_ctor_get(x_18, 2); +lean_inc(x_162); +x_163 = lean_ctor_get(x_18, 3); +lean_inc(x_163); +x_164 = lean_ctor_get(x_18, 4); +lean_inc(x_164); +lean_dec(x_18); +x_165 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__2(x_2, x_155); +if (x_165 == 0) +{ +lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; uint8_t x_175; +x_166 = lean_unsigned_to_nat(1u); +x_167 = lean_nat_add(x_140, x_166); +lean_dec(x_140); +x_168 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_168, 0, x_2); +lean_ctor_set(x_168, 1, x_161); +lean_ctor_set(x_168, 2, x_155); +x_169 = lean_array_uset(x_141, x_154, x_168); +x_170 = lean_unsigned_to_nat(4u); +x_171 = lean_nat_mul(x_167, x_170); +x_172 = lean_unsigned_to_nat(3u); +x_173 = lean_nat_div(x_171, x_172); +lean_dec(x_171); +x_174 = lean_array_get_size(x_169); +x_175 = lean_nat_dec_le(x_173, x_174); +lean_dec(x_174); +lean_dec(x_173); +if (x_175 == 0) +{ +lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; +x_176 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__3(x_169); +x_177 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_177, 0, x_167); lean_ctor_set(x_177, 1, x_176); -lean_ctor_set(x_177, 2, x_154); -lean_ctor_set(x_177, 3, x_155); -lean_ctor_set(x_177, 4, x_156); -x_178 = lean_st_ref_set(x_7, x_177, x_13); -x_179 = lean_ctor_get(x_178, 1); -lean_inc(x_179); -if (lean_is_exclusive(x_178)) { - lean_ctor_release(x_178, 0); - lean_ctor_release(x_178, 1); - x_180 = x_178; +x_178 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_178, 0, x_157); +lean_ctor_set(x_178, 1, x_177); +lean_ctor_set(x_178, 2, x_162); +lean_ctor_set(x_178, 3, x_163); +lean_ctor_set(x_178, 4, x_164); +x_179 = lean_st_ref_set(x_9, x_178, x_21); +x_180 = lean_ctor_get(x_179, 1); +lean_inc(x_180); +if (lean_is_exclusive(x_179)) { + lean_ctor_release(x_179, 0); + lean_ctor_release(x_179, 1); + x_181 = x_179; +} else { + lean_dec_ref(x_179); + x_181 = lean_box(0); +} +x_182 = lean_box(0); +if (lean_is_scalar(x_181)) { + x_183 = lean_alloc_ctor(0, 2, 0); +} else { + x_183 = x_181; +} +lean_ctor_set(x_183, 0, x_182); +lean_ctor_set(x_183, 1, x_180); +x_11 = x_183; +goto block_16; +} +else +{ +lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; +x_184 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_184, 0, x_167); +lean_ctor_set(x_184, 1, x_169); +x_185 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_185, 0, x_157); +lean_ctor_set(x_185, 1, x_184); +lean_ctor_set(x_185, 2, x_162); +lean_ctor_set(x_185, 3, x_163); +lean_ctor_set(x_185, 4, x_164); +x_186 = lean_st_ref_set(x_9, x_185, x_21); +x_187 = lean_ctor_get(x_186, 1); +lean_inc(x_187); +if (lean_is_exclusive(x_186)) { + lean_ctor_release(x_186, 0); + lean_ctor_release(x_186, 1); + x_188 = x_186; } else { - lean_dec_ref(x_178); - x_180 = lean_box(0); + lean_dec_ref(x_186); + x_188 = lean_box(0); } -x_181 = lean_box(0); -if (lean_is_scalar(x_180)) { - x_182 = lean_alloc_ctor(0, 2, 0); +x_189 = lean_box(0); +if (lean_is_scalar(x_188)) { + x_190 = lean_alloc_ctor(0, 2, 0); } else { - x_182 = x_180; -} -lean_ctor_set(x_182, 0, x_181); -lean_ctor_set(x_182, 1, x_179); -return x_182; -} -} -else -{ -lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; -x_183 = lean_box(0); -x_184 = lean_array_uset(x_133, x_146, x_183); -x_185 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__6(x_1, x_153, x_147); -x_186 = lean_array_uset(x_184, x_146, x_185); -x_187 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_187, 0, x_132); -lean_ctor_set(x_187, 1, x_186); -x_188 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_188, 0, x_149); -lean_ctor_set(x_188, 1, x_187); -lean_ctor_set(x_188, 2, x_154); -lean_ctor_set(x_188, 3, x_155); -lean_ctor_set(x_188, 4, x_156); -x_189 = lean_st_ref_set(x_7, x_188, x_13); -x_190 = lean_ctor_get(x_189, 1); -lean_inc(x_190); -if (lean_is_exclusive(x_189)) { - lean_ctor_release(x_189, 0); - lean_ctor_release(x_189, 1); - x_191 = x_189; + x_190 = x_188; +} +lean_ctor_set(x_190, 0, x_189); +lean_ctor_set(x_190, 1, x_187); +x_11 = x_190; +goto block_16; +} +} +else +{ +lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; +x_191 = lean_box(0); +x_192 = lean_array_uset(x_141, x_154, x_191); +x_193 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__6(x_2, x_161, x_155); +x_194 = lean_array_uset(x_192, x_154, x_193); +x_195 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_195, 0, x_140); +lean_ctor_set(x_195, 1, x_194); +x_196 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_196, 0, x_157); +lean_ctor_set(x_196, 1, x_195); +lean_ctor_set(x_196, 2, x_162); +lean_ctor_set(x_196, 3, x_163); +lean_ctor_set(x_196, 4, x_164); +x_197 = lean_st_ref_set(x_9, x_196, x_21); +x_198 = lean_ctor_get(x_197, 1); +lean_inc(x_198); +if (lean_is_exclusive(x_197)) { + lean_ctor_release(x_197, 0); + lean_ctor_release(x_197, 1); + x_199 = x_197; } else { - lean_dec_ref(x_189); - x_191 = lean_box(0); + lean_dec_ref(x_197); + x_199 = lean_box(0); } -x_192 = lean_box(0); -if (lean_is_scalar(x_191)) { - x_193 = lean_alloc_ctor(0, 2, 0); +x_200 = lean_box(0); +if (lean_is_scalar(x_199)) { + x_201 = lean_alloc_ctor(0, 2, 0); } else { - x_193 = x_191; + x_201 = x_199; } -lean_ctor_set(x_193, 0, x_192); -lean_ctor_set(x_193, 1, x_190); -return x_193; +lean_ctor_set(x_201, 0, x_200); +lean_ctor_set(x_201, 1, x_198); +x_11 = x_201; +goto block_16; } } else { -lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; uint8_t x_205; -lean_free_object(x_9); +lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; uint8_t x_213; +lean_free_object(x_17); +lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); -x_194 = lean_ctor_get(x_148, 0); -lean_inc(x_194); -lean_dec(x_148); -x_195 = lean_ctor_get(x_10, 0); -lean_inc(x_195); -x_196 = lean_ctor_get(x_194, 0); -lean_inc(x_196); -x_197 = lean_ctor_get(x_194, 1); -lean_inc(x_197); -x_198 = lean_ctor_get(x_194, 2); -lean_inc(x_198); -x_199 = lean_ctor_get(x_194, 3); -lean_inc(x_199); -lean_dec(x_194); -x_200 = lean_array_push(x_199, x_3); -x_201 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_201, 0, x_196); -lean_ctor_set(x_201, 1, x_197); -lean_ctor_set(x_201, 2, x_198); -lean_ctor_set(x_201, 3, x_200); -x_202 = lean_ctor_get(x_10, 2); +x_202 = lean_ctor_get(x_156, 0); lean_inc(x_202); -x_203 = lean_ctor_get(x_10, 3); +lean_dec(x_156); +x_203 = lean_ctor_get(x_18, 0); lean_inc(x_203); -x_204 = lean_ctor_get(x_10, 4); +x_204 = lean_ctor_get(x_202, 0); lean_inc(x_204); -lean_dec(x_10); -x_205 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__2(x_1, x_147); -if (x_205 == 0) -{ -lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; uint8_t x_215; -x_206 = lean_unsigned_to_nat(1u); -x_207 = lean_nat_add(x_132, x_206); -lean_dec(x_132); -x_208 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_208, 0, x_1); -lean_ctor_set(x_208, 1, x_201); -lean_ctor_set(x_208, 2, x_147); -x_209 = lean_array_uset(x_133, x_146, x_208); -x_210 = lean_unsigned_to_nat(4u); -x_211 = lean_nat_mul(x_207, x_210); -x_212 = lean_unsigned_to_nat(3u); -x_213 = lean_nat_div(x_211, x_212); -lean_dec(x_211); -x_214 = lean_array_get_size(x_209); -x_215 = lean_nat_dec_le(x_213, x_214); -lean_dec(x_214); -lean_dec(x_213); -if (x_215 == 0) -{ -lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; -x_216 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__3(x_209); -x_217 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_217, 0, x_207); -lean_ctor_set(x_217, 1, x_216); -x_218 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_218, 0, x_195); -lean_ctor_set(x_218, 1, x_217); -lean_ctor_set(x_218, 2, x_202); -lean_ctor_set(x_218, 3, x_203); -lean_ctor_set(x_218, 4, x_204); -x_219 = lean_st_ref_set(x_7, x_218, x_13); -x_220 = lean_ctor_get(x_219, 1); -lean_inc(x_220); -if (lean_is_exclusive(x_219)) { - lean_ctor_release(x_219, 0); - lean_ctor_release(x_219, 1); - x_221 = x_219; -} else { - lean_dec_ref(x_219); - x_221 = lean_box(0); -} -x_222 = lean_box(0); -if (lean_is_scalar(x_221)) { - x_223 = lean_alloc_ctor(0, 2, 0); -} else { - x_223 = x_221; -} -lean_ctor_set(x_223, 0, x_222); -lean_ctor_set(x_223, 1, x_220); -return x_223; -} -else +x_205 = lean_ctor_get(x_202, 1); +lean_inc(x_205); +x_206 = lean_ctor_get(x_202, 2); +lean_inc(x_206); +x_207 = lean_ctor_get(x_202, 3); +lean_inc(x_207); +lean_dec(x_202); +x_208 = lean_array_push(x_207, x_4); +x_209 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_209, 0, x_204); +lean_ctor_set(x_209, 1, x_205); +lean_ctor_set(x_209, 2, x_206); +lean_ctor_set(x_209, 3, x_208); +x_210 = lean_ctor_get(x_18, 2); +lean_inc(x_210); +x_211 = lean_ctor_get(x_18, 3); +lean_inc(x_211); +x_212 = lean_ctor_get(x_18, 4); +lean_inc(x_212); +lean_dec(x_18); +x_213 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__2(x_2, x_155); +if (x_213 == 0) +{ +lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; uint8_t x_223; +x_214 = lean_unsigned_to_nat(1u); +x_215 = lean_nat_add(x_140, x_214); +lean_dec(x_140); +x_216 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_216, 0, x_2); +lean_ctor_set(x_216, 1, x_209); +lean_ctor_set(x_216, 2, x_155); +x_217 = lean_array_uset(x_141, x_154, x_216); +x_218 = lean_unsigned_to_nat(4u); +x_219 = lean_nat_mul(x_215, x_218); +x_220 = lean_unsigned_to_nat(3u); +x_221 = lean_nat_div(x_219, x_220); +lean_dec(x_219); +x_222 = lean_array_get_size(x_217); +x_223 = lean_nat_dec_le(x_221, x_222); +lean_dec(x_222); +lean_dec(x_221); +if (x_223 == 0) { -lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; -x_224 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_224, 0, x_207); -lean_ctor_set(x_224, 1, x_209); -x_225 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_225, 0, x_195); +lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; +x_224 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__3(x_217); +x_225 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_225, 0, x_215); lean_ctor_set(x_225, 1, x_224); -lean_ctor_set(x_225, 2, x_202); -lean_ctor_set(x_225, 3, x_203); -lean_ctor_set(x_225, 4, x_204); -x_226 = lean_st_ref_set(x_7, x_225, x_13); -x_227 = lean_ctor_get(x_226, 1); -lean_inc(x_227); -if (lean_is_exclusive(x_226)) { - lean_ctor_release(x_226, 0); - lean_ctor_release(x_226, 1); - x_228 = x_226; +x_226 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_226, 0, x_203); +lean_ctor_set(x_226, 1, x_225); +lean_ctor_set(x_226, 2, x_210); +lean_ctor_set(x_226, 3, x_211); +lean_ctor_set(x_226, 4, x_212); +x_227 = lean_st_ref_set(x_9, x_226, x_21); +x_228 = lean_ctor_get(x_227, 1); +lean_inc(x_228); +if (lean_is_exclusive(x_227)) { + lean_ctor_release(x_227, 0); + lean_ctor_release(x_227, 1); + x_229 = x_227; } else { - lean_dec_ref(x_226); - x_228 = lean_box(0); + lean_dec_ref(x_227); + x_229 = lean_box(0); } -x_229 = lean_box(0); -if (lean_is_scalar(x_228)) { - x_230 = lean_alloc_ctor(0, 2, 0); +x_230 = lean_box(0); +if (lean_is_scalar(x_229)) { + x_231 = lean_alloc_ctor(0, 2, 0); } else { - x_230 = x_228; -} -lean_ctor_set(x_230, 0, x_229); -lean_ctor_set(x_230, 1, x_227); -return x_230; -} + x_231 = x_229; +} +lean_ctor_set(x_231, 0, x_230); +lean_ctor_set(x_231, 1, x_228); +x_11 = x_231; +goto block_16; +} +else +{ +lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; +x_232 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_232, 0, x_215); +lean_ctor_set(x_232, 1, x_217); +x_233 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_233, 0, x_203); +lean_ctor_set(x_233, 1, x_232); +lean_ctor_set(x_233, 2, x_210); +lean_ctor_set(x_233, 3, x_211); +lean_ctor_set(x_233, 4, x_212); +x_234 = lean_st_ref_set(x_9, x_233, x_21); +x_235 = lean_ctor_get(x_234, 1); +lean_inc(x_235); +if (lean_is_exclusive(x_234)) { + lean_ctor_release(x_234, 0); + lean_ctor_release(x_234, 1); + x_236 = x_234; +} else { + lean_dec_ref(x_234); + x_236 = lean_box(0); } -else -{ -lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; -x_231 = lean_box(0); -x_232 = lean_array_uset(x_133, x_146, x_231); -x_233 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__6(x_1, x_201, x_147); -x_234 = lean_array_uset(x_232, x_146, x_233); -x_235 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_235, 0, x_132); -lean_ctor_set(x_235, 1, x_234); -x_236 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_236, 0, x_195); -lean_ctor_set(x_236, 1, x_235); -lean_ctor_set(x_236, 2, x_202); -lean_ctor_set(x_236, 3, x_203); -lean_ctor_set(x_236, 4, x_204); -x_237 = lean_st_ref_set(x_7, x_236, x_13); -x_238 = lean_ctor_get(x_237, 1); -lean_inc(x_238); -if (lean_is_exclusive(x_237)) { - lean_ctor_release(x_237, 0); - lean_ctor_release(x_237, 1); - x_239 = x_237; +x_237 = lean_box(0); +if (lean_is_scalar(x_236)) { + x_238 = lean_alloc_ctor(0, 2, 0); +} else { + x_238 = x_236; +} +lean_ctor_set(x_238, 0, x_237); +lean_ctor_set(x_238, 1, x_235); +x_11 = x_238; +goto block_16; +} +} +else +{ +lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; +x_239 = lean_box(0); +x_240 = lean_array_uset(x_141, x_154, x_239); +x_241 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__6(x_2, x_209, x_155); +x_242 = lean_array_uset(x_240, x_154, x_241); +x_243 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_243, 0, x_140); +lean_ctor_set(x_243, 1, x_242); +x_244 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_244, 0, x_203); +lean_ctor_set(x_244, 1, x_243); +lean_ctor_set(x_244, 2, x_210); +lean_ctor_set(x_244, 3, x_211); +lean_ctor_set(x_244, 4, x_212); +x_245 = lean_st_ref_set(x_9, x_244, x_21); +x_246 = lean_ctor_get(x_245, 1); +lean_inc(x_246); +if (lean_is_exclusive(x_245)) { + lean_ctor_release(x_245, 0); + lean_ctor_release(x_245, 1); + x_247 = x_245; } else { - lean_dec_ref(x_237); - x_239 = lean_box(0); + lean_dec_ref(x_245); + x_247 = lean_box(0); } -x_240 = lean_box(0); -if (lean_is_scalar(x_239)) { - x_241 = lean_alloc_ctor(0, 2, 0); +x_248 = lean_box(0); +if (lean_is_scalar(x_247)) { + x_249 = lean_alloc_ctor(0, 2, 0); } else { - x_241 = x_239; + x_249 = x_247; } -lean_ctor_set(x_241, 0, x_240); -lean_ctor_set(x_241, 1, x_238); -return x_241; +lean_ctor_set(x_249, 0, x_248); +lean_ctor_set(x_249, 1, x_246); +x_11 = x_249; +goto block_16; } } } } else { -lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; uint64_t x_247; uint64_t x_248; uint64_t x_249; uint64_t x_250; uint64_t x_251; uint64_t x_252; uint64_t x_253; size_t x_254; size_t x_255; size_t x_256; size_t x_257; size_t x_258; lean_object* x_259; lean_object* x_260; -x_242 = lean_ctor_get(x_9, 1); -lean_inc(x_242); -lean_dec(x_9); -x_243 = lean_ctor_get(x_11, 0); -lean_inc(x_243); -x_244 = lean_ctor_get(x_11, 1); -lean_inc(x_244); -if (lean_is_exclusive(x_11)) { - lean_ctor_release(x_11, 0); - lean_ctor_release(x_11, 1); - x_245 = x_11; +lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; uint64_t x_255; uint64_t x_256; uint64_t x_257; uint64_t x_258; uint64_t x_259; uint64_t x_260; uint64_t x_261; size_t x_262; size_t x_263; size_t x_264; size_t x_265; size_t x_266; lean_object* x_267; lean_object* x_268; +x_250 = lean_ctor_get(x_17, 1); +lean_inc(x_250); +lean_dec(x_17); +x_251 = lean_ctor_get(x_19, 0); +lean_inc(x_251); +x_252 = lean_ctor_get(x_19, 1); +lean_inc(x_252); +if (lean_is_exclusive(x_19)) { + lean_ctor_release(x_19, 0); + lean_ctor_release(x_19, 1); + x_253 = x_19; } else { - lean_dec_ref(x_11); - x_245 = lean_box(0); -} -x_246 = lean_array_get_size(x_244); -x_247 = l___private_Lean_Syntax_0__String_hashRange____x40_Lean_Syntax___hyg_169_(x_1); -x_248 = 32; -x_249 = lean_uint64_shift_right(x_247, x_248); -x_250 = lean_uint64_xor(x_247, x_249); -x_251 = 16; -x_252 = lean_uint64_shift_right(x_250, x_251); -x_253 = lean_uint64_xor(x_250, x_252); -x_254 = lean_uint64_to_usize(x_253); -x_255 = lean_usize_of_nat(x_246); -lean_dec(x_246); -x_256 = 1; -x_257 = lean_usize_sub(x_255, x_256); -x_258 = lean_usize_land(x_254, x_257); -x_259 = lean_array_uget(x_244, x_258); -x_260 = l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_collectReferences___spec__1(x_1, x_259); -if (lean_obj_tag(x_260) == 0) -{ -lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; uint8_t x_270; -x_261 = lean_ctor_get(x_10, 0); -lean_inc(x_261); -x_262 = l_Lean_LocalDecl_userName(x_2); -x_263 = lean_box(0); -x_264 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_264, 0, x_3); -lean_ctor_set(x_264, 1, x_263); -x_265 = lean_array_mk(x_264); -x_266 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_266, 0, x_262); -lean_ctor_set(x_266, 1, x_4); -lean_ctor_set(x_266, 2, x_5); -lean_ctor_set(x_266, 3, x_265); -x_267 = lean_ctor_get(x_10, 2); -lean_inc(x_267); -x_268 = lean_ctor_get(x_10, 3); -lean_inc(x_268); -x_269 = lean_ctor_get(x_10, 4); + lean_dec_ref(x_19); + x_253 = lean_box(0); +} +x_254 = lean_array_get_size(x_252); +x_255 = l___private_Lean_Syntax_0__String_hashRange____x40_Lean_Syntax___hyg_169_(x_2); +x_256 = 32; +x_257 = lean_uint64_shift_right(x_255, x_256); +x_258 = lean_uint64_xor(x_255, x_257); +x_259 = 16; +x_260 = lean_uint64_shift_right(x_258, x_259); +x_261 = lean_uint64_xor(x_258, x_260); +x_262 = lean_uint64_to_usize(x_261); +x_263 = lean_usize_of_nat(x_254); +lean_dec(x_254); +x_264 = 1; +x_265 = lean_usize_sub(x_263, x_264); +x_266 = lean_usize_land(x_262, x_265); +x_267 = lean_array_uget(x_252, x_266); +x_268 = l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__1(x_2, x_267); +if (lean_obj_tag(x_268) == 0) +{ +lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; uint8_t x_278; +x_269 = lean_ctor_get(x_18, 0); lean_inc(x_269); -lean_dec(x_10); -x_270 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__2(x_1, x_259); -if (x_270 == 0) +x_270 = l_Lean_LocalDecl_userName(x_3); +x_271 = lean_box(0); +x_272 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_272, 0, x_4); +lean_ctor_set(x_272, 1, x_271); +x_273 = lean_array_mk(x_272); +x_274 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_274, 0, x_270); +lean_ctor_set(x_274, 1, x_5); +lean_ctor_set(x_274, 2, x_6); +lean_ctor_set(x_274, 3, x_273); +x_275 = lean_ctor_get(x_18, 2); +lean_inc(x_275); +x_276 = lean_ctor_get(x_18, 3); +lean_inc(x_276); +x_277 = lean_ctor_get(x_18, 4); +lean_inc(x_277); +lean_dec(x_18); +x_278 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__2(x_2, x_267); +if (x_278 == 0) +{ +lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; lean_object* x_286; lean_object* x_287; uint8_t x_288; +x_279 = lean_unsigned_to_nat(1u); +x_280 = lean_nat_add(x_251, x_279); +lean_dec(x_251); +x_281 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_281, 0, x_2); +lean_ctor_set(x_281, 1, x_274); +lean_ctor_set(x_281, 2, x_267); +x_282 = lean_array_uset(x_252, x_266, x_281); +x_283 = lean_unsigned_to_nat(4u); +x_284 = lean_nat_mul(x_280, x_283); +x_285 = lean_unsigned_to_nat(3u); +x_286 = lean_nat_div(x_284, x_285); +lean_dec(x_284); +x_287 = lean_array_get_size(x_282); +x_288 = lean_nat_dec_le(x_286, x_287); +lean_dec(x_287); +lean_dec(x_286); +if (x_288 == 0) { -lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; uint8_t x_280; -x_271 = lean_unsigned_to_nat(1u); -x_272 = lean_nat_add(x_243, x_271); -lean_dec(x_243); -x_273 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_273, 0, x_1); -lean_ctor_set(x_273, 1, x_266); -lean_ctor_set(x_273, 2, x_259); -x_274 = lean_array_uset(x_244, x_258, x_273); -x_275 = lean_unsigned_to_nat(4u); -x_276 = lean_nat_mul(x_272, x_275); -x_277 = lean_unsigned_to_nat(3u); -x_278 = lean_nat_div(x_276, x_277); -lean_dec(x_276); -x_279 = lean_array_get_size(x_274); -x_280 = lean_nat_dec_le(x_278, x_279); -lean_dec(x_279); -lean_dec(x_278); -if (x_280 == 0) -{ -lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; lean_object* x_286; lean_object* x_287; lean_object* x_288; -x_281 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__3(x_274); -if (lean_is_scalar(x_245)) { - x_282 = lean_alloc_ctor(0, 2, 0); +lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; lean_object* x_294; lean_object* x_295; lean_object* x_296; +x_289 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__3(x_282); +if (lean_is_scalar(x_253)) { + x_290 = lean_alloc_ctor(0, 2, 0); } else { - x_282 = x_245; -} -lean_ctor_set(x_282, 0, x_272); -lean_ctor_set(x_282, 1, x_281); -x_283 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_283, 0, x_261); -lean_ctor_set(x_283, 1, x_282); -lean_ctor_set(x_283, 2, x_267); -lean_ctor_set(x_283, 3, x_268); -lean_ctor_set(x_283, 4, x_269); -x_284 = lean_st_ref_set(x_7, x_283, x_242); -x_285 = lean_ctor_get(x_284, 1); -lean_inc(x_285); -if (lean_is_exclusive(x_284)) { - lean_ctor_release(x_284, 0); - lean_ctor_release(x_284, 1); - x_286 = x_284; + x_290 = x_253; +} +lean_ctor_set(x_290, 0, x_280); +lean_ctor_set(x_290, 1, x_289); +x_291 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_291, 0, x_269); +lean_ctor_set(x_291, 1, x_290); +lean_ctor_set(x_291, 2, x_275); +lean_ctor_set(x_291, 3, x_276); +lean_ctor_set(x_291, 4, x_277); +x_292 = lean_st_ref_set(x_9, x_291, x_250); +x_293 = lean_ctor_get(x_292, 1); +lean_inc(x_293); +if (lean_is_exclusive(x_292)) { + lean_ctor_release(x_292, 0); + lean_ctor_release(x_292, 1); + x_294 = x_292; } else { - lean_dec_ref(x_284); - x_286 = lean_box(0); + lean_dec_ref(x_292); + x_294 = lean_box(0); } -x_287 = lean_box(0); -if (lean_is_scalar(x_286)) { - x_288 = lean_alloc_ctor(0, 2, 0); +x_295 = lean_box(0); +if (lean_is_scalar(x_294)) { + x_296 = lean_alloc_ctor(0, 2, 0); } else { - x_288 = x_286; + x_296 = x_294; } -lean_ctor_set(x_288, 0, x_287); -lean_ctor_set(x_288, 1, x_285); -return x_288; +lean_ctor_set(x_296, 0, x_295); +lean_ctor_set(x_296, 1, x_293); +x_11 = x_296; +goto block_16; } else { -lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; lean_object* x_294; lean_object* x_295; -if (lean_is_scalar(x_245)) { - x_289 = lean_alloc_ctor(0, 2, 0); +lean_object* x_297; lean_object* x_298; lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; lean_object* x_303; +if (lean_is_scalar(x_253)) { + x_297 = lean_alloc_ctor(0, 2, 0); } else { - x_289 = x_245; -} -lean_ctor_set(x_289, 0, x_272); -lean_ctor_set(x_289, 1, x_274); -x_290 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_290, 0, x_261); -lean_ctor_set(x_290, 1, x_289); -lean_ctor_set(x_290, 2, x_267); -lean_ctor_set(x_290, 3, x_268); -lean_ctor_set(x_290, 4, x_269); -x_291 = lean_st_ref_set(x_7, x_290, x_242); -x_292 = lean_ctor_get(x_291, 1); -lean_inc(x_292); -if (lean_is_exclusive(x_291)) { - lean_ctor_release(x_291, 0); - lean_ctor_release(x_291, 1); - x_293 = x_291; + x_297 = x_253; +} +lean_ctor_set(x_297, 0, x_280); +lean_ctor_set(x_297, 1, x_282); +x_298 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_298, 0, x_269); +lean_ctor_set(x_298, 1, x_297); +lean_ctor_set(x_298, 2, x_275); +lean_ctor_set(x_298, 3, x_276); +lean_ctor_set(x_298, 4, x_277); +x_299 = lean_st_ref_set(x_9, x_298, x_250); +x_300 = lean_ctor_get(x_299, 1); +lean_inc(x_300); +if (lean_is_exclusive(x_299)) { + lean_ctor_release(x_299, 0); + lean_ctor_release(x_299, 1); + x_301 = x_299; } else { - lean_dec_ref(x_291); - x_293 = lean_box(0); + lean_dec_ref(x_299); + x_301 = lean_box(0); } -x_294 = lean_box(0); -if (lean_is_scalar(x_293)) { - x_295 = lean_alloc_ctor(0, 2, 0); +x_302 = lean_box(0); +if (lean_is_scalar(x_301)) { + x_303 = lean_alloc_ctor(0, 2, 0); } else { - x_295 = x_293; + x_303 = x_301; } -lean_ctor_set(x_295, 0, x_294); -lean_ctor_set(x_295, 1, x_292); -return x_295; +lean_ctor_set(x_303, 0, x_302); +lean_ctor_set(x_303, 1, x_300); +x_11 = x_303; +goto block_16; } } else { -lean_object* x_296; lean_object* x_297; lean_object* x_298; lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; -x_296 = lean_box(0); -x_297 = lean_array_uset(x_244, x_258, x_296); -x_298 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__6(x_1, x_266, x_259); -x_299 = lean_array_uset(x_297, x_258, x_298); -if (lean_is_scalar(x_245)) { - x_300 = lean_alloc_ctor(0, 2, 0); +lean_object* x_304; lean_object* x_305; lean_object* x_306; lean_object* x_307; lean_object* x_308; lean_object* x_309; lean_object* x_310; lean_object* x_311; lean_object* x_312; lean_object* x_313; lean_object* x_314; +x_304 = lean_box(0); +x_305 = lean_array_uset(x_252, x_266, x_304); +x_306 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__6(x_2, x_274, x_267); +x_307 = lean_array_uset(x_305, x_266, x_306); +if (lean_is_scalar(x_253)) { + x_308 = lean_alloc_ctor(0, 2, 0); } else { - x_300 = x_245; -} -lean_ctor_set(x_300, 0, x_243); -lean_ctor_set(x_300, 1, x_299); -x_301 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_301, 0, x_261); -lean_ctor_set(x_301, 1, x_300); -lean_ctor_set(x_301, 2, x_267); -lean_ctor_set(x_301, 3, x_268); -lean_ctor_set(x_301, 4, x_269); -x_302 = lean_st_ref_set(x_7, x_301, x_242); -x_303 = lean_ctor_get(x_302, 1); -lean_inc(x_303); -if (lean_is_exclusive(x_302)) { - lean_ctor_release(x_302, 0); - lean_ctor_release(x_302, 1); - x_304 = x_302; + x_308 = x_253; +} +lean_ctor_set(x_308, 0, x_251); +lean_ctor_set(x_308, 1, x_307); +x_309 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_309, 0, x_269); +lean_ctor_set(x_309, 1, x_308); +lean_ctor_set(x_309, 2, x_275); +lean_ctor_set(x_309, 3, x_276); +lean_ctor_set(x_309, 4, x_277); +x_310 = lean_st_ref_set(x_9, x_309, x_250); +x_311 = lean_ctor_get(x_310, 1); +lean_inc(x_311); +if (lean_is_exclusive(x_310)) { + lean_ctor_release(x_310, 0); + lean_ctor_release(x_310, 1); + x_312 = x_310; } else { - lean_dec_ref(x_302); - x_304 = lean_box(0); + lean_dec_ref(x_310); + x_312 = lean_box(0); } -x_305 = lean_box(0); -if (lean_is_scalar(x_304)) { - x_306 = lean_alloc_ctor(0, 2, 0); +x_313 = lean_box(0); +if (lean_is_scalar(x_312)) { + x_314 = lean_alloc_ctor(0, 2, 0); } else { - x_306 = x_304; + x_314 = x_312; } -lean_ctor_set(x_306, 0, x_305); -lean_ctor_set(x_306, 1, x_303); -return x_306; +lean_ctor_set(x_314, 0, x_313); +lean_ctor_set(x_314, 1, x_311); +x_11 = x_314; +goto block_16; } } else { -lean_object* x_307; lean_object* x_308; lean_object* x_309; lean_object* x_310; lean_object* x_311; lean_object* x_312; lean_object* x_313; lean_object* x_314; lean_object* x_315; lean_object* x_316; lean_object* x_317; uint8_t x_318; +lean_object* x_315; lean_object* x_316; lean_object* x_317; lean_object* x_318; lean_object* x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; lean_object* x_324; lean_object* x_325; uint8_t x_326; +lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); -x_307 = lean_ctor_get(x_260, 0); -lean_inc(x_307); -lean_dec(x_260); -x_308 = lean_ctor_get(x_10, 0); -lean_inc(x_308); -x_309 = lean_ctor_get(x_307, 0); -lean_inc(x_309); -x_310 = lean_ctor_get(x_307, 1); -lean_inc(x_310); -x_311 = lean_ctor_get(x_307, 2); -lean_inc(x_311); -x_312 = lean_ctor_get(x_307, 3); -lean_inc(x_312); -lean_dec(x_307); -x_313 = lean_array_push(x_312, x_3); -x_314 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_314, 0, x_309); -lean_ctor_set(x_314, 1, x_310); -lean_ctor_set(x_314, 2, x_311); -lean_ctor_set(x_314, 3, x_313); -x_315 = lean_ctor_get(x_10, 2); +x_315 = lean_ctor_get(x_268, 0); lean_inc(x_315); -x_316 = lean_ctor_get(x_10, 3); +lean_dec(x_268); +x_316 = lean_ctor_get(x_18, 0); lean_inc(x_316); -x_317 = lean_ctor_get(x_10, 4); +x_317 = lean_ctor_get(x_315, 0); lean_inc(x_317); -lean_dec(x_10); -x_318 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__2(x_1, x_259); -if (x_318 == 0) +x_318 = lean_ctor_get(x_315, 1); +lean_inc(x_318); +x_319 = lean_ctor_get(x_315, 2); +lean_inc(x_319); +x_320 = lean_ctor_get(x_315, 3); +lean_inc(x_320); +lean_dec(x_315); +x_321 = lean_array_push(x_320, x_4); +x_322 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_322, 0, x_317); +lean_ctor_set(x_322, 1, x_318); +lean_ctor_set(x_322, 2, x_319); +lean_ctor_set(x_322, 3, x_321); +x_323 = lean_ctor_get(x_18, 2); +lean_inc(x_323); +x_324 = lean_ctor_get(x_18, 3); +lean_inc(x_324); +x_325 = lean_ctor_get(x_18, 4); +lean_inc(x_325); +lean_dec(x_18); +x_326 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__2(x_2, x_267); +if (x_326 == 0) { -lean_object* x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; lean_object* x_324; lean_object* x_325; lean_object* x_326; lean_object* x_327; uint8_t x_328; -x_319 = lean_unsigned_to_nat(1u); -x_320 = lean_nat_add(x_243, x_319); -lean_dec(x_243); -x_321 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_321, 0, x_1); -lean_ctor_set(x_321, 1, x_314); -lean_ctor_set(x_321, 2, x_259); -x_322 = lean_array_uset(x_244, x_258, x_321); -x_323 = lean_unsigned_to_nat(4u); -x_324 = lean_nat_mul(x_320, x_323); -x_325 = lean_unsigned_to_nat(3u); -x_326 = lean_nat_div(x_324, x_325); -lean_dec(x_324); -x_327 = lean_array_get_size(x_322); -x_328 = lean_nat_dec_le(x_326, x_327); -lean_dec(x_327); -lean_dec(x_326); -if (x_328 == 0) -{ -lean_object* x_329; lean_object* x_330; lean_object* x_331; lean_object* x_332; lean_object* x_333; lean_object* x_334; lean_object* x_335; lean_object* x_336; -x_329 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__3(x_322); -if (lean_is_scalar(x_245)) { - x_330 = lean_alloc_ctor(0, 2, 0); +lean_object* x_327; lean_object* x_328; lean_object* x_329; lean_object* x_330; lean_object* x_331; lean_object* x_332; lean_object* x_333; lean_object* x_334; lean_object* x_335; uint8_t x_336; +x_327 = lean_unsigned_to_nat(1u); +x_328 = lean_nat_add(x_251, x_327); +lean_dec(x_251); +x_329 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_329, 0, x_2); +lean_ctor_set(x_329, 1, x_322); +lean_ctor_set(x_329, 2, x_267); +x_330 = lean_array_uset(x_252, x_266, x_329); +x_331 = lean_unsigned_to_nat(4u); +x_332 = lean_nat_mul(x_328, x_331); +x_333 = lean_unsigned_to_nat(3u); +x_334 = lean_nat_div(x_332, x_333); +lean_dec(x_332); +x_335 = lean_array_get_size(x_330); +x_336 = lean_nat_dec_le(x_334, x_335); +lean_dec(x_335); +lean_dec(x_334); +if (x_336 == 0) +{ +lean_object* x_337; lean_object* x_338; lean_object* x_339; lean_object* x_340; lean_object* x_341; lean_object* x_342; lean_object* x_343; lean_object* x_344; +x_337 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__3(x_330); +if (lean_is_scalar(x_253)) { + x_338 = lean_alloc_ctor(0, 2, 0); } else { - x_330 = x_245; -} -lean_ctor_set(x_330, 0, x_320); -lean_ctor_set(x_330, 1, x_329); -x_331 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_331, 0, x_308); -lean_ctor_set(x_331, 1, x_330); -lean_ctor_set(x_331, 2, x_315); -lean_ctor_set(x_331, 3, x_316); -lean_ctor_set(x_331, 4, x_317); -x_332 = lean_st_ref_set(x_7, x_331, x_242); -x_333 = lean_ctor_get(x_332, 1); -lean_inc(x_333); -if (lean_is_exclusive(x_332)) { - lean_ctor_release(x_332, 0); - lean_ctor_release(x_332, 1); - x_334 = x_332; + x_338 = x_253; +} +lean_ctor_set(x_338, 0, x_328); +lean_ctor_set(x_338, 1, x_337); +x_339 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_339, 0, x_316); +lean_ctor_set(x_339, 1, x_338); +lean_ctor_set(x_339, 2, x_323); +lean_ctor_set(x_339, 3, x_324); +lean_ctor_set(x_339, 4, x_325); +x_340 = lean_st_ref_set(x_9, x_339, x_250); +x_341 = lean_ctor_get(x_340, 1); +lean_inc(x_341); +if (lean_is_exclusive(x_340)) { + lean_ctor_release(x_340, 0); + lean_ctor_release(x_340, 1); + x_342 = x_340; } else { - lean_dec_ref(x_332); - x_334 = lean_box(0); + lean_dec_ref(x_340); + x_342 = lean_box(0); } -x_335 = lean_box(0); -if (lean_is_scalar(x_334)) { - x_336 = lean_alloc_ctor(0, 2, 0); +x_343 = lean_box(0); +if (lean_is_scalar(x_342)) { + x_344 = lean_alloc_ctor(0, 2, 0); } else { - x_336 = x_334; + x_344 = x_342; } -lean_ctor_set(x_336, 0, x_335); -lean_ctor_set(x_336, 1, x_333); -return x_336; +lean_ctor_set(x_344, 0, x_343); +lean_ctor_set(x_344, 1, x_341); +x_11 = x_344; +goto block_16; } else { -lean_object* x_337; lean_object* x_338; lean_object* x_339; lean_object* x_340; lean_object* x_341; lean_object* x_342; lean_object* x_343; -if (lean_is_scalar(x_245)) { - x_337 = lean_alloc_ctor(0, 2, 0); +lean_object* x_345; lean_object* x_346; lean_object* x_347; lean_object* x_348; lean_object* x_349; lean_object* x_350; lean_object* x_351; +if (lean_is_scalar(x_253)) { + x_345 = lean_alloc_ctor(0, 2, 0); } else { - x_337 = x_245; -} -lean_ctor_set(x_337, 0, x_320); -lean_ctor_set(x_337, 1, x_322); -x_338 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_338, 0, x_308); -lean_ctor_set(x_338, 1, x_337); -lean_ctor_set(x_338, 2, x_315); -lean_ctor_set(x_338, 3, x_316); -lean_ctor_set(x_338, 4, x_317); -x_339 = lean_st_ref_set(x_7, x_338, x_242); -x_340 = lean_ctor_get(x_339, 1); -lean_inc(x_340); -if (lean_is_exclusive(x_339)) { - lean_ctor_release(x_339, 0); - lean_ctor_release(x_339, 1); - x_341 = x_339; + x_345 = x_253; +} +lean_ctor_set(x_345, 0, x_328); +lean_ctor_set(x_345, 1, x_330); +x_346 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_346, 0, x_316); +lean_ctor_set(x_346, 1, x_345); +lean_ctor_set(x_346, 2, x_323); +lean_ctor_set(x_346, 3, x_324); +lean_ctor_set(x_346, 4, x_325); +x_347 = lean_st_ref_set(x_9, x_346, x_250); +x_348 = lean_ctor_get(x_347, 1); +lean_inc(x_348); +if (lean_is_exclusive(x_347)) { + lean_ctor_release(x_347, 0); + lean_ctor_release(x_347, 1); + x_349 = x_347; } else { - lean_dec_ref(x_339); - x_341 = lean_box(0); + lean_dec_ref(x_347); + x_349 = lean_box(0); } -x_342 = lean_box(0); -if (lean_is_scalar(x_341)) { - x_343 = lean_alloc_ctor(0, 2, 0); +x_350 = lean_box(0); +if (lean_is_scalar(x_349)) { + x_351 = lean_alloc_ctor(0, 2, 0); } else { - x_343 = x_341; + x_351 = x_349; } -lean_ctor_set(x_343, 0, x_342); -lean_ctor_set(x_343, 1, x_340); -return x_343; +lean_ctor_set(x_351, 0, x_350); +lean_ctor_set(x_351, 1, x_348); +x_11 = x_351; +goto block_16; } } else { -lean_object* x_344; lean_object* x_345; lean_object* x_346; lean_object* x_347; lean_object* x_348; lean_object* x_349; lean_object* x_350; lean_object* x_351; lean_object* x_352; lean_object* x_353; lean_object* x_354; -x_344 = lean_box(0); -x_345 = lean_array_uset(x_244, x_258, x_344); -x_346 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__6(x_1, x_314, x_259); -x_347 = lean_array_uset(x_345, x_258, x_346); -if (lean_is_scalar(x_245)) { - x_348 = lean_alloc_ctor(0, 2, 0); +lean_object* x_352; lean_object* x_353; lean_object* x_354; lean_object* x_355; lean_object* x_356; lean_object* x_357; lean_object* x_358; lean_object* x_359; lean_object* x_360; lean_object* x_361; lean_object* x_362; +x_352 = lean_box(0); +x_353 = lean_array_uset(x_252, x_266, x_352); +x_354 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__6(x_2, x_322, x_267); +x_355 = lean_array_uset(x_353, x_266, x_354); +if (lean_is_scalar(x_253)) { + x_356 = lean_alloc_ctor(0, 2, 0); } else { - x_348 = x_245; -} -lean_ctor_set(x_348, 0, x_243); -lean_ctor_set(x_348, 1, x_347); -x_349 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_349, 0, x_308); -lean_ctor_set(x_349, 1, x_348); -lean_ctor_set(x_349, 2, x_315); -lean_ctor_set(x_349, 3, x_316); -lean_ctor_set(x_349, 4, x_317); -x_350 = lean_st_ref_set(x_7, x_349, x_242); -x_351 = lean_ctor_get(x_350, 1); -lean_inc(x_351); -if (lean_is_exclusive(x_350)) { - lean_ctor_release(x_350, 0); - lean_ctor_release(x_350, 1); - x_352 = x_350; + x_356 = x_253; +} +lean_ctor_set(x_356, 0, x_251); +lean_ctor_set(x_356, 1, x_355); +x_357 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_357, 0, x_316); +lean_ctor_set(x_357, 1, x_356); +lean_ctor_set(x_357, 2, x_323); +lean_ctor_set(x_357, 3, x_324); +lean_ctor_set(x_357, 4, x_325); +x_358 = lean_st_ref_set(x_9, x_357, x_250); +x_359 = lean_ctor_get(x_358, 1); +lean_inc(x_359); +if (lean_is_exclusive(x_358)) { + lean_ctor_release(x_358, 0); + lean_ctor_release(x_358, 1); + x_360 = x_358; } else { - lean_dec_ref(x_350); - x_352 = lean_box(0); + lean_dec_ref(x_358); + x_360 = lean_box(0); } -x_353 = lean_box(0); -if (lean_is_scalar(x_352)) { - x_354 = lean_alloc_ctor(0, 2, 0); +x_361 = lean_box(0); +if (lean_is_scalar(x_360)) { + x_362 = lean_alloc_ctor(0, 2, 0); } else { - x_354 = x_352; + x_362 = x_360; } -lean_ctor_set(x_354, 0, x_353); -lean_ctor_set(x_354, 1, x_351); -return x_354; +lean_ctor_set(x_362, 0, x_361); +lean_ctor_set(x_362, 1, x_359); +x_11 = x_362; +goto block_16; } } } +block_16: +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +x_14 = lean_box(x_8); +x_15 = lean_apply_4(x_1, x_12, x_14, x_9, x_13); +return x_15; +} } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__1() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__1() { _start: { lean_object* x_1; @@ -11715,31 +12316,31 @@ x_1 = lean_mk_string_unchecked("_", 1, 1); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__2() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__1; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__1; x_2 = lean_string_length(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__3() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__1; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__1; x_2 = lean_string_utf8_byte_size(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__4() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__1; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__1; x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__3; +x_3 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__3; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -11747,3902 +12348,5156 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, uint8_t x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_9; lean_object* x_10; -x_9 = l_Lean_Linter_UnusedVariables_collectReferences_skipDeclIdIfPresent(x_1); -x_10 = l_Lean_Syntax_getId(x_9); -if (lean_obj_tag(x_10) == 1) +lean_object* x_11; lean_object* x_12; +x_11 = l_Lean_Linter_UnusedVariables_collectReferences_skipDeclIdIfPresent(x_1); +x_12 = l_Lean_Syntax_getId(x_11); +if (lean_obj_tag(x_12) == 1) { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; -x_11 = lean_ctor_get(x_10, 1); -lean_inc(x_11); -lean_dec(x_10); -x_12 = lean_string_utf8_byte_size(x_11); -x_13 = lean_unsigned_to_nat(0u); -lean_inc(x_11); -x_14 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_14, 0, x_11); -lean_ctor_set(x_14, 1, x_13); -lean_ctor_set(x_14, 2, x_12); -x_15 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__2; -x_16 = l_Substring_nextn(x_14, x_15, x_13); -lean_dec(x_14); -x_17 = lean_nat_add(x_13, x_16); +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; +x_13 = lean_ctor_get(x_12, 1); +lean_inc(x_13); +lean_dec(x_12); +x_14 = lean_string_utf8_byte_size(x_13); +x_15 = lean_unsigned_to_nat(0u); +lean_inc(x_13); +x_16 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_16, 0, x_13); +lean_ctor_set(x_16, 1, x_15); +lean_ctor_set(x_16, 2, x_14); +x_17 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__2; +x_18 = l_Substring_nextn(x_16, x_17, x_15); lean_dec(x_16); -x_18 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_18, 0, x_11); -lean_ctor_set(x_18, 1, x_13); -lean_ctor_set(x_18, 2, x_17); -x_19 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__4; -x_20 = l_Substring_beq(x_18, x_19); -if (x_20 == 0) +x_19 = lean_nat_add(x_15, x_18); +lean_dec(x_18); +x_20 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_20, 0, x_13); +lean_ctor_set(x_20, 1, x_15); +lean_ctor_set(x_20, 2, x_19); +x_21 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__4; +x_22 = l_Substring_beq(x_20, x_21); +if (x_22 == 0) { -lean_object* x_21; lean_object* x_22; -x_21 = lean_box(0); -x_22 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__1(x_2, x_3, x_4, x_9, x_5, x_21, x_7, x_8); -return x_22; +lean_object* x_23; lean_object* x_24; +x_23 = lean_box(0); +x_24 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__3(x_2, x_3, x_4, x_5, x_11, x_6, x_23, x_8, x_9, x_10); +return x_24; } else { -lean_object* x_23; lean_object* x_24; +uint8_t x_25; lean_object* x_26; lean_object* x_27; +lean_dec(x_11); lean_dec(x_9); +lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); -x_23 = lean_box(0); -x_24 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_24, 0, x_23); -lean_ctor_set(x_24, 1, x_8); -return x_24; +x_25 = 1; +x_26 = lean_box(x_25); +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_10); +return x_27; } } else { -lean_object* x_25; lean_object* x_26; -lean_dec(x_10); -x_25 = lean_box(0); -x_26 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__1(x_2, x_3, x_4, x_9, x_5, x_25, x_7, x_8); -return x_26; +lean_object* x_28; lean_object* x_29; +lean_dec(x_12); +x_28 = lean_box(0); +x_29 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__3(x_2, x_3, x_4, x_5, x_11, x_6, x_28, x_8, x_9, x_10); +return x_29; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, uint8_t x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_9 = lean_ctor_get(x_1, 0); -lean_inc(x_9); +lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); lean_dec(x_1); -x_10 = lean_ctor_get(x_9, 3); -lean_inc(x_10); -lean_dec(x_9); -x_11 = l_Lean_Linter_getLinterUnusedVariables___closed__1; -x_12 = l_Lean_Linter_getLinterValue(x_11, x_10); -if (x_12 == 0) +x_12 = lean_ctor_get(x_11, 3); +lean_inc(x_12); +lean_dec(x_11); +x_13 = l_Lean_Linter_getLinterUnusedVariables___closed__1; +x_14 = l_Lean_Linter_getLinterValue(x_13, x_12); +if (x_14 == 0) { -lean_object* x_13; lean_object* x_14; -lean_dec(x_10); -lean_dec(x_5); +uint8_t x_15; lean_object* x_16; lean_object* x_17; +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_13 = lean_box(0); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_13); -lean_ctor_set(x_14, 1, x_8); -return x_14; +x_15 = 1; +x_16 = lean_box(x_15); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_16); +lean_ctor_set(x_17, 1, x_10); +return x_17; } else { -lean_object* x_15; lean_object* x_16; -x_15 = lean_box(0); -x_16 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2(x_2, x_3, x_4, x_5, x_10, x_15, x_7, x_8); -return x_16; +lean_object* x_18; lean_object* x_19; +x_18 = lean_box(0); +x_19 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4(x_2, x_3, x_4, x_5, x_6, x_12, x_18, x_8, x_9, x_10); +return x_19; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, uint8_t x_9, lean_object* x_10, lean_object* x_11) { _start: { -switch (lean_obj_tag(x_3)) { -case 0: +lean_object* x_12; lean_object* x_13; +x_12 = lean_ctor_get(x_1, 1); +lean_inc(x_12); +lean_dec(x_1); +lean_inc(x_2); +x_13 = lean_local_ctx_find(x_12, x_2); +if (lean_obj_tag(x_13) == 0) { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; -lean_dec(x_2); -x_7 = lean_ctor_get(x_3, 0); -lean_inc(x_7); +uint8_t x_14; lean_object* x_15; lean_object* x_16; +lean_dec(x_10); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); -x_8 = lean_st_ref_take(x_5, x_6); -x_9 = lean_ctor_get(x_8, 0); -lean_inc(x_9); -x_10 = lean_ctor_get(x_8, 1); -lean_inc(x_10); -lean_dec(x_8); -x_11 = !lean_is_exclusive(x_9); -if (x_11 == 0) +lean_dec(x_2); +x_14 = 1; +x_15 = lean_box(x_14); +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_16, 1, x_11); +return x_16; +} +else { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; -x_12 = lean_ctor_get(x_9, 4); -x_13 = lean_ctor_get(x_7, 3); -lean_inc(x_13); -lean_dec(x_7); -x_14 = lean_ctor_get(x_13, 7); -lean_inc(x_14); +lean_object* x_17; lean_object* x_18; uint8_t x_19; uint8_t x_20; +x_17 = lean_ctor_get(x_13, 0); +lean_inc(x_17); lean_dec(x_13); -x_15 = lean_array_push(x_12, x_14); -lean_ctor_set(x_9, 4, x_15); -x_16 = lean_st_ref_set(x_5, x_9, x_10); -x_17 = !lean_is_exclusive(x_16); -if (x_17 == 0) -{ -lean_object* x_18; lean_object* x_19; -x_18 = lean_ctor_get(x_16, 0); +x_18 = lean_ctor_get(x_6, 0); +lean_inc(x_18); +x_19 = 0; +x_20 = l_String_Range_contains(x_7, x_18, x_19); lean_dec(x_18); -x_19 = lean_box(0); -lean_ctor_set(x_16, 0, x_19); -return x_16; +if (x_20 == 0) +{ +uint8_t x_21; lean_object* x_22; lean_object* x_23; +lean_dec(x_17); +lean_dec(x_10); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_21 = 1; +x_22 = lean_box(x_21); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_11); +return x_23; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_16, 1); -lean_inc(x_20); -lean_dec(x_16); -x_21 = lean_box(0); -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_21); -lean_ctor_set(x_22, 1, x_20); -return x_22; -} +lean_object* x_24; uint8_t x_25; +x_24 = l_Lean_LocalDecl_userName(x_17); +x_25 = l_Lean_Name_hasMacroScopes(x_24); +lean_dec(x_24); +if (x_25 == 0) +{ +lean_object* x_26; lean_object* x_27; +x_26 = lean_box(0); +x_27 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__5(x_3, x_4, x_5, x_6, x_17, x_2, x_26, x_9, x_10, x_11); +lean_dec(x_17); +return x_27; } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_23 = lean_ctor_get(x_9, 0); -x_24 = lean_ctor_get(x_9, 1); -x_25 = lean_ctor_get(x_9, 2); -x_26 = lean_ctor_get(x_9, 3); -x_27 = lean_ctor_get(x_9, 4); -lean_inc(x_27); -lean_inc(x_26); -lean_inc(x_25); -lean_inc(x_24); -lean_inc(x_23); -lean_dec(x_9); -x_28 = lean_ctor_get(x_7, 3); -lean_inc(x_28); -lean_dec(x_7); -x_29 = lean_ctor_get(x_28, 7); -lean_inc(x_29); -lean_dec(x_28); -x_30 = lean_array_push(x_27, x_29); -x_31 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_31, 0, x_23); -lean_ctor_set(x_31, 1, x_24); -lean_ctor_set(x_31, 2, x_25); -lean_ctor_set(x_31, 3, x_26); -lean_ctor_set(x_31, 4, x_30); -x_32 = lean_st_ref_set(x_5, x_31, x_10); -x_33 = lean_ctor_get(x_32, 1); -lean_inc(x_33); -if (lean_is_exclusive(x_32)) { - lean_ctor_release(x_32, 0); - lean_ctor_release(x_32, 1); - x_34 = x_32; -} else { - lean_dec_ref(x_32); - x_34 = lean_box(0); +uint8_t x_28; lean_object* x_29; lean_object* x_30; +lean_dec(x_17); +lean_dec(x_10); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_28 = 1; +x_29 = lean_box(x_28); +x_30 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_30, 0, x_29); +lean_ctor_set(x_30, 1, x_11); +return x_30; } -x_35 = lean_box(0); -if (lean_is_scalar(x_34)) { - x_36 = lean_alloc_ctor(0, 2, 0); -} else { - x_36 = x_34; } -lean_ctor_set(x_36, 0, x_35); -lean_ctor_set(x_36, 1, x_33); -return x_36; } } -case 1: +} +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__7___closed__1() { +_start: { -lean_object* x_37; lean_object* x_38; -x_37 = lean_ctor_get(x_3, 0); -lean_inc(x_37); -x_38 = lean_ctor_get(x_37, 3); -lean_inc(x_38); -switch (lean_obj_tag(x_38)) { +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__2___boxed), 4, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__7(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, uint8_t x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; +x_10 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__7___closed__1; +x_11 = lean_ctor_get(x_1, 3); +lean_inc(x_11); +switch (lean_obj_tag(x_11)) { case 1: { -lean_object* x_39; lean_object* x_40; -x_39 = lean_ctor_get(x_38, 0); -lean_inc(x_39); -lean_dec(x_38); -x_40 = l_Lean_Elab_Info_range_x3f(x_3); -if (lean_obj_tag(x_40) == 0) +lean_object* x_12; lean_object* x_13; +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +lean_dec(x_11); +x_13 = l_Lean_Elab_Info_range_x3f(x_2); +if (lean_obj_tag(x_13) == 0) { -lean_object* x_41; lean_object* x_42; -lean_dec(x_39); -lean_dec(x_37); -lean_dec(x_3); -lean_dec(x_2); -x_41 = lean_box(0); -x_42 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_42, 0, x_41); -lean_ctor_set(x_42, 1, x_6); -return x_42; +uint8_t x_14; lean_object* x_15; lean_object* x_16; +lean_dec(x_12); +lean_dec(x_8); +lean_dec(x_4); +lean_dec(x_1); +x_14 = 1; +x_15 = lean_box(x_14); +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_16, 1, x_9); +return x_16; } else { -lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_43 = lean_ctor_get(x_40, 0); -lean_inc(x_43); -lean_dec(x_40); -x_44 = l_Lean_Elab_Info_stx(x_3); -lean_dec(x_3); -x_45 = l_Lean_Syntax_getHeadInfo(x_44); -if (lean_obj_tag(x_45) == 0) +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_13, 0); +lean_inc(x_17); +lean_dec(x_13); +x_18 = l_Lean_Elab_Info_stx(x_2); +x_19 = l_Lean_Syntax_getHeadInfo(x_18); +if (lean_obj_tag(x_19) == 0) { -uint8_t x_46; -lean_dec(x_45); -x_46 = lean_ctor_get_uint8(x_37, sizeof(void*)*4); -if (x_46 == 0) +uint8_t x_20; +lean_dec(x_19); +x_20 = lean_ctor_get_uint8(x_1, sizeof(void*)*4); +if (x_20 == 0) { -lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; uint8_t x_55; -lean_dec(x_44); -lean_dec(x_43); -lean_dec(x_37); -lean_dec(x_2); -x_47 = lean_st_ref_take(x_5, x_6); -x_48 = lean_ctor_get(x_47, 0); -lean_inc(x_48); -x_49 = lean_ctor_get(x_48, 2); -lean_inc(x_49); -x_50 = lean_ctor_get(x_47, 1); -lean_inc(x_50); -lean_dec(x_47); -x_51 = lean_ctor_get(x_48, 0); -lean_inc(x_51); -x_52 = lean_ctor_get(x_48, 1); -lean_inc(x_52); -x_53 = lean_ctor_get(x_48, 3); -lean_inc(x_53); -x_54 = lean_ctor_get(x_48, 4); -lean_inc(x_54); -lean_dec(x_48); -x_55 = !lean_is_exclusive(x_49); -if (x_55 == 0) +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_4); +lean_dec(x_1); +x_21 = lean_st_ref_take(x_8, x_9); +x_22 = lean_ctor_get(x_21, 0); +lean_inc(x_22); +x_23 = lean_ctor_get(x_22, 2); +lean_inc(x_23); +x_24 = lean_ctor_get(x_21, 1); +lean_inc(x_24); +lean_dec(x_21); +x_25 = lean_ctor_get(x_22, 0); +lean_inc(x_25); +x_26 = lean_ctor_get(x_22, 1); +lean_inc(x_26); +x_27 = lean_ctor_get(x_22, 3); +lean_inc(x_27); +x_28 = lean_ctor_get(x_22, 4); +lean_inc(x_28); +lean_dec(x_22); +x_29 = !lean_is_exclusive(x_23); +if (x_29 == 0) { -lean_object* x_56; lean_object* x_57; lean_object* x_58; uint64_t x_59; uint64_t x_60; uint64_t x_61; uint64_t x_62; uint64_t x_63; uint64_t x_64; uint64_t x_65; size_t x_66; size_t x_67; size_t x_68; size_t x_69; size_t x_70; lean_object* x_71; uint8_t x_72; -x_56 = lean_ctor_get(x_49, 0); -x_57 = lean_ctor_get(x_49, 1); -x_58 = lean_array_get_size(x_57); -x_59 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_39); -x_60 = 32; -x_61 = lean_uint64_shift_right(x_59, x_60); -x_62 = lean_uint64_xor(x_59, x_61); -x_63 = 16; -x_64 = lean_uint64_shift_right(x_62, x_63); -x_65 = lean_uint64_xor(x_62, x_64); -x_66 = lean_uint64_to_usize(x_65); -x_67 = lean_usize_of_nat(x_58); -lean_dec(x_58); -x_68 = 1; -x_69 = lean_usize_sub(x_67, x_68); -x_70 = lean_usize_land(x_66, x_69); -x_71 = lean_array_uget(x_57, x_70); -x_72 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_39, x_71); -if (x_72 == 0) -{ -lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; uint8_t x_83; -x_73 = lean_unsigned_to_nat(1u); -x_74 = lean_nat_add(x_56, x_73); +lean_object* x_30; lean_object* x_31; lean_object* x_32; uint64_t x_33; uint64_t x_34; uint64_t x_35; uint64_t x_36; uint64_t x_37; uint64_t x_38; uint64_t x_39; size_t x_40; size_t x_41; size_t x_42; size_t x_43; size_t x_44; lean_object* x_45; uint8_t x_46; +x_30 = lean_ctor_get(x_23, 0); +x_31 = lean_ctor_get(x_23, 1); +x_32 = lean_array_get_size(x_31); +x_33 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_12); +x_34 = 32; +x_35 = lean_uint64_shift_right(x_33, x_34); +x_36 = lean_uint64_xor(x_33, x_35); +x_37 = 16; +x_38 = lean_uint64_shift_right(x_36, x_37); +x_39 = lean_uint64_xor(x_36, x_38); +x_40 = lean_uint64_to_usize(x_39); +x_41 = lean_usize_of_nat(x_32); +lean_dec(x_32); +x_42 = 1; +x_43 = lean_usize_sub(x_41, x_42); +x_44 = lean_usize_land(x_40, x_43); +x_45 = lean_array_uget(x_31, x_44); +x_46 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_12, x_45); +if (x_46 == 0) +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; uint8_t x_57; +x_47 = lean_unsigned_to_nat(1u); +x_48 = lean_nat_add(x_30, x_47); +lean_dec(x_30); +x_49 = lean_box(0); +x_50 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_50, 0, x_12); +lean_ctor_set(x_50, 1, x_49); +lean_ctor_set(x_50, 2, x_45); +x_51 = lean_array_uset(x_31, x_44, x_50); +x_52 = lean_unsigned_to_nat(4u); +x_53 = lean_nat_mul(x_48, x_52); +x_54 = lean_unsigned_to_nat(3u); +x_55 = lean_nat_div(x_53, x_54); +lean_dec(x_53); +x_56 = lean_array_get_size(x_51); +x_57 = lean_nat_dec_le(x_55, x_56); lean_dec(x_56); -x_75 = lean_box(0); -x_76 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_76, 0, x_39); -lean_ctor_set(x_76, 1, x_75); -lean_ctor_set(x_76, 2, x_71); -x_77 = lean_array_uset(x_57, x_70, x_76); -x_78 = lean_unsigned_to_nat(4u); -x_79 = lean_nat_mul(x_74, x_78); -x_80 = lean_unsigned_to_nat(3u); -x_81 = lean_nat_div(x_79, x_80); -lean_dec(x_79); -x_82 = lean_array_get_size(x_77); -x_83 = lean_nat_dec_le(x_81, x_82); -lean_dec(x_82); -lean_dec(x_81); -if (x_83 == 0) +lean_dec(x_55); +if (x_57 == 0) { -lean_object* x_84; lean_object* x_85; lean_object* x_86; uint8_t x_87; -x_84 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_77); -lean_ctor_set(x_49, 1, x_84); -lean_ctor_set(x_49, 0, x_74); -x_85 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_85, 0, x_51); -lean_ctor_set(x_85, 1, x_52); -lean_ctor_set(x_85, 2, x_49); -lean_ctor_set(x_85, 3, x_53); -lean_ctor_set(x_85, 4, x_54); -x_86 = lean_st_ref_set(x_5, x_85, x_50); -x_87 = !lean_is_exclusive(x_86); -if (x_87 == 0) -{ -lean_object* x_88; -x_88 = lean_ctor_get(x_86, 0); -lean_dec(x_88); -lean_ctor_set(x_86, 0, x_75); -return x_86; +lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; +x_58 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_51); +lean_ctor_set(x_23, 1, x_58); +lean_ctor_set(x_23, 0, x_48); +x_59 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_59, 0, x_25); +lean_ctor_set(x_59, 1, x_26); +lean_ctor_set(x_59, 2, x_23); +lean_ctor_set(x_59, 3, x_27); +lean_ctor_set(x_59, 4, x_28); +x_60 = lean_st_ref_set(x_8, x_59, x_24); +x_61 = lean_ctor_get(x_60, 1); +lean_inc(x_61); +lean_dec(x_60); +x_62 = lean_box(x_7); +x_63 = lean_apply_4(x_10, x_49, x_62, x_8, x_61); +return x_63; } else { -lean_object* x_89; lean_object* x_90; -x_89 = lean_ctor_get(x_86, 1); -lean_inc(x_89); -lean_dec(x_86); -x_90 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_90, 0, x_75); -lean_ctor_set(x_90, 1, x_89); -return x_90; +lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; +lean_ctor_set(x_23, 1, x_51); +lean_ctor_set(x_23, 0, x_48); +x_64 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_64, 0, x_25); +lean_ctor_set(x_64, 1, x_26); +lean_ctor_set(x_64, 2, x_23); +lean_ctor_set(x_64, 3, x_27); +lean_ctor_set(x_64, 4, x_28); +x_65 = lean_st_ref_set(x_8, x_64, x_24); +x_66 = lean_ctor_get(x_65, 1); +lean_inc(x_66); +lean_dec(x_65); +x_67 = lean_box(x_7); +x_68 = lean_apply_4(x_10, x_49, x_67, x_8, x_66); +return x_68; } } else { -lean_object* x_91; lean_object* x_92; uint8_t x_93; -lean_ctor_set(x_49, 1, x_77); -lean_ctor_set(x_49, 0, x_74); -x_91 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_91, 0, x_51); -lean_ctor_set(x_91, 1, x_52); -lean_ctor_set(x_91, 2, x_49); -lean_ctor_set(x_91, 3, x_53); -lean_ctor_set(x_91, 4, x_54); -x_92 = lean_st_ref_set(x_5, x_91, x_50); -x_93 = !lean_is_exclusive(x_92); -if (x_93 == 0) +lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; +lean_dec(x_45); +lean_dec(x_12); +x_69 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_69, 0, x_25); +lean_ctor_set(x_69, 1, x_26); +lean_ctor_set(x_69, 2, x_23); +lean_ctor_set(x_69, 3, x_27); +lean_ctor_set(x_69, 4, x_28); +x_70 = lean_st_ref_set(x_8, x_69, x_24); +x_71 = lean_ctor_get(x_70, 1); +lean_inc(x_71); +lean_dec(x_70); +x_72 = lean_box(0); +x_73 = lean_box(x_7); +x_74 = lean_apply_4(x_10, x_72, x_73, x_8, x_71); +return x_74; +} +} +else { -lean_object* x_94; -x_94 = lean_ctor_get(x_92, 0); -lean_dec(x_94); -lean_ctor_set(x_92, 0, x_75); -return x_92; +lean_object* x_75; lean_object* x_76; lean_object* x_77; uint64_t x_78; uint64_t x_79; uint64_t x_80; uint64_t x_81; uint64_t x_82; uint64_t x_83; uint64_t x_84; size_t x_85; size_t x_86; size_t x_87; size_t x_88; size_t x_89; lean_object* x_90; uint8_t x_91; +x_75 = lean_ctor_get(x_23, 0); +x_76 = lean_ctor_get(x_23, 1); +lean_inc(x_76); +lean_inc(x_75); +lean_dec(x_23); +x_77 = lean_array_get_size(x_76); +x_78 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_12); +x_79 = 32; +x_80 = lean_uint64_shift_right(x_78, x_79); +x_81 = lean_uint64_xor(x_78, x_80); +x_82 = 16; +x_83 = lean_uint64_shift_right(x_81, x_82); +x_84 = lean_uint64_xor(x_81, x_83); +x_85 = lean_uint64_to_usize(x_84); +x_86 = lean_usize_of_nat(x_77); +lean_dec(x_77); +x_87 = 1; +x_88 = lean_usize_sub(x_86, x_87); +x_89 = lean_usize_land(x_85, x_88); +x_90 = lean_array_uget(x_76, x_89); +x_91 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_12, x_90); +if (x_91 == 0) +{ +lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; uint8_t x_102; +x_92 = lean_unsigned_to_nat(1u); +x_93 = lean_nat_add(x_75, x_92); +lean_dec(x_75); +x_94 = lean_box(0); +x_95 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_95, 0, x_12); +lean_ctor_set(x_95, 1, x_94); +lean_ctor_set(x_95, 2, x_90); +x_96 = lean_array_uset(x_76, x_89, x_95); +x_97 = lean_unsigned_to_nat(4u); +x_98 = lean_nat_mul(x_93, x_97); +x_99 = lean_unsigned_to_nat(3u); +x_100 = lean_nat_div(x_98, x_99); +lean_dec(x_98); +x_101 = lean_array_get_size(x_96); +x_102 = lean_nat_dec_le(x_100, x_101); +lean_dec(x_101); +lean_dec(x_100); +if (x_102 == 0) +{ +lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; +x_103 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_96); +x_104 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_104, 0, x_93); +lean_ctor_set(x_104, 1, x_103); +x_105 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_105, 0, x_25); +lean_ctor_set(x_105, 1, x_26); +lean_ctor_set(x_105, 2, x_104); +lean_ctor_set(x_105, 3, x_27); +lean_ctor_set(x_105, 4, x_28); +x_106 = lean_st_ref_set(x_8, x_105, x_24); +x_107 = lean_ctor_get(x_106, 1); +lean_inc(x_107); +lean_dec(x_106); +x_108 = lean_box(x_7); +x_109 = lean_apply_4(x_10, x_94, x_108, x_8, x_107); +return x_109; } else { -lean_object* x_95; lean_object* x_96; -x_95 = lean_ctor_get(x_92, 1); -lean_inc(x_95); -lean_dec(x_92); -x_96 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_96, 0, x_75); -lean_ctor_set(x_96, 1, x_95); -return x_96; +lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; +x_110 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_110, 0, x_93); +lean_ctor_set(x_110, 1, x_96); +x_111 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_111, 0, x_25); +lean_ctor_set(x_111, 1, x_26); +lean_ctor_set(x_111, 2, x_110); +lean_ctor_set(x_111, 3, x_27); +lean_ctor_set(x_111, 4, x_28); +x_112 = lean_st_ref_set(x_8, x_111, x_24); +x_113 = lean_ctor_get(x_112, 1); +lean_inc(x_113); +lean_dec(x_112); +x_114 = lean_box(x_7); +x_115 = lean_apply_4(x_10, x_94, x_114, x_8, x_113); +return x_115; +} +} +else +{ +lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; +lean_dec(x_90); +lean_dec(x_12); +x_116 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_116, 0, x_75); +lean_ctor_set(x_116, 1, x_76); +x_117 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_117, 0, x_25); +lean_ctor_set(x_117, 1, x_26); +lean_ctor_set(x_117, 2, x_116); +lean_ctor_set(x_117, 3, x_27); +lean_ctor_set(x_117, 4, x_28); +x_118 = lean_st_ref_set(x_8, x_117, x_24); +x_119 = lean_ctor_get(x_118, 1); +lean_inc(x_119); +lean_dec(x_118); +x_120 = lean_box(0); +x_121 = lean_box(x_7); +x_122 = lean_apply_4(x_10, x_120, x_121, x_8, x_119); +return x_122; } } } else { -lean_object* x_97; lean_object* x_98; uint8_t x_99; -lean_dec(x_71); -lean_dec(x_39); -x_97 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_97, 0, x_51); -lean_ctor_set(x_97, 1, x_52); -lean_ctor_set(x_97, 2, x_49); -lean_ctor_set(x_97, 3, x_53); -lean_ctor_set(x_97, 4, x_54); -x_98 = lean_st_ref_set(x_5, x_97, x_50); -x_99 = !lean_is_exclusive(x_98); -if (x_99 == 0) +if (x_3 == 0) { -lean_object* x_100; lean_object* x_101; -x_100 = lean_ctor_get(x_98, 0); -lean_dec(x_100); -x_101 = lean_box(0); -lean_ctor_set(x_98, 0, x_101); -return x_98; +lean_object* x_123; lean_object* x_124; +x_123 = lean_box(0); +x_124 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__6(x_1, x_12, x_4, x_18, x_10, x_17, x_5, x_123, x_7, x_8, x_9); +return x_124; } else { -lean_object* x_102; lean_object* x_103; lean_object* x_104; -x_102 = lean_ctor_get(x_98, 1); -lean_inc(x_102); -lean_dec(x_98); -x_103 = lean_box(0); -x_104 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_104, 0, x_103); -lean_ctor_set(x_104, 1, x_102); -return x_104; +uint8_t x_125; lean_object* x_126; lean_object* x_127; +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_12); +lean_dec(x_8); +lean_dec(x_4); +lean_dec(x_1); +x_125 = 1; +x_126 = lean_box(x_125); +x_127 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_127, 0, x_126); +lean_ctor_set(x_127, 1, x_9); +return x_127; } } } else { -lean_object* x_105; lean_object* x_106; lean_object* x_107; uint64_t x_108; uint64_t x_109; uint64_t x_110; uint64_t x_111; uint64_t x_112; uint64_t x_113; uint64_t x_114; size_t x_115; size_t x_116; size_t x_117; size_t x_118; size_t x_119; lean_object* x_120; uint8_t x_121; -x_105 = lean_ctor_get(x_49, 0); -x_106 = lean_ctor_get(x_49, 1); -lean_inc(x_106); -lean_inc(x_105); -lean_dec(x_49); -x_107 = lean_array_get_size(x_106); -x_108 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_39); -x_109 = 32; -x_110 = lean_uint64_shift_right(x_108, x_109); -x_111 = lean_uint64_xor(x_108, x_110); -x_112 = 16; -x_113 = lean_uint64_shift_right(x_111, x_112); -x_114 = lean_uint64_xor(x_111, x_113); -x_115 = lean_uint64_to_usize(x_114); -x_116 = lean_usize_of_nat(x_107); -lean_dec(x_107); -x_117 = 1; -x_118 = lean_usize_sub(x_116, x_117); -x_119 = lean_usize_land(x_115, x_118); -x_120 = lean_array_uget(x_106, x_119); -x_121 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_39, x_120); -if (x_121 == 0) -{ -lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; uint8_t x_132; -x_122 = lean_unsigned_to_nat(1u); -x_123 = lean_nat_add(x_105, x_122); -lean_dec(x_105); -x_124 = lean_box(0); -x_125 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_125, 0, x_39); -lean_ctor_set(x_125, 1, x_124); -lean_ctor_set(x_125, 2, x_120); -x_126 = lean_array_uset(x_106, x_119, x_125); -x_127 = lean_unsigned_to_nat(4u); -x_128 = lean_nat_mul(x_123, x_127); -x_129 = lean_unsigned_to_nat(3u); -x_130 = lean_nat_div(x_128, x_129); -lean_dec(x_128); -x_131 = lean_array_get_size(x_126); -x_132 = lean_nat_dec_le(x_130, x_131); -lean_dec(x_131); -lean_dec(x_130); -if (x_132 == 0) -{ -lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; -x_133 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_126); -x_134 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_134, 0, x_123); -lean_ctor_set(x_134, 1, x_133); -x_135 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_135, 0, x_51); -lean_ctor_set(x_135, 1, x_52); -lean_ctor_set(x_135, 2, x_134); -lean_ctor_set(x_135, 3, x_53); -lean_ctor_set(x_135, 4, x_54); -x_136 = lean_st_ref_set(x_5, x_135, x_50); -x_137 = lean_ctor_get(x_136, 1); -lean_inc(x_137); -if (lean_is_exclusive(x_136)) { - lean_ctor_release(x_136, 0); - lean_ctor_release(x_136, 1); - x_138 = x_136; -} else { - lean_dec_ref(x_136); - x_138 = lean_box(0); -} -if (lean_is_scalar(x_138)) { - x_139 = lean_alloc_ctor(0, 2, 0); -} else { - x_139 = x_138; -} -lean_ctor_set(x_139, 0, x_124); -lean_ctor_set(x_139, 1, x_137); -return x_139; -} -else -{ -lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; -x_140 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_140, 0, x_123); -lean_ctor_set(x_140, 1, x_126); -x_141 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_141, 0, x_51); -lean_ctor_set(x_141, 1, x_52); -lean_ctor_set(x_141, 2, x_140); -lean_ctor_set(x_141, 3, x_53); -lean_ctor_set(x_141, 4, x_54); -x_142 = lean_st_ref_set(x_5, x_141, x_50); -x_143 = lean_ctor_get(x_142, 1); -lean_inc(x_143); -if (lean_is_exclusive(x_142)) { - lean_ctor_release(x_142, 0); - lean_ctor_release(x_142, 1); - x_144 = x_142; -} else { - lean_dec_ref(x_142); - x_144 = lean_box(0); +uint8_t x_128; lean_object* x_129; lean_object* x_130; +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_12); +lean_dec(x_8); +lean_dec(x_4); +lean_dec(x_1); +x_128 = 1; +x_129 = lean_box(x_128); +x_130 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_130, 0, x_129); +lean_ctor_set(x_130, 1, x_9); +return x_130; } -if (lean_is_scalar(x_144)) { - x_145 = lean_alloc_ctor(0, 2, 0); -} else { - x_145 = x_144; } -lean_ctor_set(x_145, 0, x_124); -lean_ctor_set(x_145, 1, x_143); -return x_145; } +case 4: +{ +uint8_t x_131; +lean_dec(x_11); +lean_dec(x_4); +x_131 = lean_ctor_get_uint8(x_1, sizeof(void*)*4); +lean_dec(x_1); +if (x_131 == 0) +{ +lean_object* x_132; lean_object* x_133; lean_object* x_134; +x_132 = lean_box(0); +x_133 = lean_box(x_7); +x_134 = lean_apply_4(x_10, x_132, x_133, x_8, x_9); +return x_134; } else { -lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; -lean_dec(x_120); -lean_dec(x_39); -x_146 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_146, 0, x_105); -lean_ctor_set(x_146, 1, x_106); -x_147 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_147, 0, x_51); -lean_ctor_set(x_147, 1, x_52); -lean_ctor_set(x_147, 2, x_146); -lean_ctor_set(x_147, 3, x_53); -lean_ctor_set(x_147, 4, x_54); -x_148 = lean_st_ref_set(x_5, x_147, x_50); -x_149 = lean_ctor_get(x_148, 1); +lean_object* x_135; +x_135 = l_Lean_Elab_Info_range_x3f(x_2); +if (lean_obj_tag(x_135) == 0) +{ +uint8_t x_136; lean_object* x_137; lean_object* x_138; +lean_dec(x_8); +x_136 = 1; +x_137 = lean_box(x_136); +x_138 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_138, 0, x_137); +lean_ctor_set(x_138, 1, x_9); +return x_138; +} +else +{ +lean_object* x_139; lean_object* x_140; lean_object* x_141; +x_139 = lean_ctor_get(x_135, 0); +lean_inc(x_139); +lean_dec(x_135); +x_140 = l_Lean_Elab_Info_stx(x_2); +x_141 = l_Lean_Syntax_getHeadInfo(x_140); +lean_dec(x_140); +if (lean_obj_tag(x_141) == 0) +{ +lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; uint8_t x_150; +lean_dec(x_141); +x_142 = lean_st_ref_take(x_8, x_9); +x_143 = lean_ctor_get(x_142, 0); +lean_inc(x_143); +x_144 = lean_ctor_get(x_143, 0); +lean_inc(x_144); +x_145 = lean_ctor_get(x_142, 1); +lean_inc(x_145); +lean_dec(x_142); +x_146 = lean_ctor_get(x_143, 1); +lean_inc(x_146); +x_147 = lean_ctor_get(x_143, 2); +lean_inc(x_147); +x_148 = lean_ctor_get(x_143, 3); +lean_inc(x_148); +x_149 = lean_ctor_get(x_143, 4); lean_inc(x_149); -if (lean_is_exclusive(x_148)) { - lean_ctor_release(x_148, 0); - lean_ctor_release(x_148, 1); - x_150 = x_148; -} else { - lean_dec_ref(x_148); - x_150 = lean_box(0); -} -x_151 = lean_box(0); -if (lean_is_scalar(x_150)) { - x_152 = lean_alloc_ctor(0, 2, 0); -} else { - x_152 = x_150; -} -lean_ctor_set(x_152, 0, x_151); -lean_ctor_set(x_152, 1, x_149); -return x_152; -} +lean_dec(x_143); +x_150 = !lean_is_exclusive(x_144); +if (x_150 == 0) +{ +lean_object* x_151; lean_object* x_152; lean_object* x_153; uint64_t x_154; uint64_t x_155; uint64_t x_156; uint64_t x_157; uint64_t x_158; uint64_t x_159; uint64_t x_160; size_t x_161; size_t x_162; size_t x_163; size_t x_164; size_t x_165; lean_object* x_166; uint8_t x_167; +x_151 = lean_ctor_get(x_144, 0); +x_152 = lean_ctor_get(x_144, 1); +x_153 = lean_array_get_size(x_152); +x_154 = l___private_Lean_Syntax_0__String_hashRange____x40_Lean_Syntax___hyg_169_(x_139); +x_155 = 32; +x_156 = lean_uint64_shift_right(x_154, x_155); +x_157 = lean_uint64_xor(x_154, x_156); +x_158 = 16; +x_159 = lean_uint64_shift_right(x_157, x_158); +x_160 = lean_uint64_xor(x_157, x_159); +x_161 = lean_uint64_to_usize(x_160); +x_162 = lean_usize_of_nat(x_153); +lean_dec(x_153); +x_163 = 1; +x_164 = lean_usize_sub(x_162, x_163); +x_165 = lean_usize_land(x_161, x_164); +x_166 = lean_array_uget(x_152, x_165); +x_167 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__7(x_139, x_166); +if (x_167 == 0) +{ +lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; uint8_t x_178; +x_168 = lean_unsigned_to_nat(1u); +x_169 = lean_nat_add(x_151, x_168); +lean_dec(x_151); +x_170 = lean_box(0); +x_171 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_171, 0, x_139); +lean_ctor_set(x_171, 1, x_170); +lean_ctor_set(x_171, 2, x_166); +x_172 = lean_array_uset(x_152, x_165, x_171); +x_173 = lean_unsigned_to_nat(4u); +x_174 = lean_nat_mul(x_169, x_173); +x_175 = lean_unsigned_to_nat(3u); +x_176 = lean_nat_div(x_174, x_175); +lean_dec(x_174); +x_177 = lean_array_get_size(x_172); +x_178 = lean_nat_dec_le(x_176, x_177); +lean_dec(x_177); +lean_dec(x_176); +if (x_178 == 0) +{ +lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; +x_179 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__8(x_172); +lean_ctor_set(x_144, 1, x_179); +lean_ctor_set(x_144, 0, x_169); +x_180 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_180, 0, x_144); +lean_ctor_set(x_180, 1, x_146); +lean_ctor_set(x_180, 2, x_147); +lean_ctor_set(x_180, 3, x_148); +lean_ctor_set(x_180, 4, x_149); +x_181 = lean_st_ref_set(x_8, x_180, x_145); +x_182 = lean_ctor_get(x_181, 1); +lean_inc(x_182); +lean_dec(x_181); +x_183 = lean_box(x_7); +x_184 = lean_apply_4(x_10, x_170, x_183, x_8, x_182); +return x_184; +} +else +{ +lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; +lean_ctor_set(x_144, 1, x_172); +lean_ctor_set(x_144, 0, x_169); +x_185 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_185, 0, x_144); +lean_ctor_set(x_185, 1, x_146); +lean_ctor_set(x_185, 2, x_147); +lean_ctor_set(x_185, 3, x_148); +lean_ctor_set(x_185, 4, x_149); +x_186 = lean_st_ref_set(x_8, x_185, x_145); +x_187 = lean_ctor_get(x_186, 1); +lean_inc(x_187); +lean_dec(x_186); +x_188 = lean_box(x_7); +x_189 = lean_apply_4(x_10, x_170, x_188, x_8, x_187); +return x_189; } } else { -lean_object* x_153; lean_object* x_154; -x_153 = lean_ctor_get(x_37, 1); -lean_inc(x_153); -lean_dec(x_37); -lean_inc(x_39); -x_154 = lean_local_ctx_find(x_153, x_39); -if (lean_obj_tag(x_154) == 0) -{ -lean_object* x_155; lean_object* x_156; -lean_dec(x_44); -lean_dec(x_43); -lean_dec(x_39); -lean_dec(x_2); -x_155 = lean_box(0); -x_156 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_156, 0, x_155); -lean_ctor_set(x_156, 1, x_6); -return x_156; +lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; +lean_dec(x_166); +lean_dec(x_139); +x_190 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_190, 0, x_144); +lean_ctor_set(x_190, 1, x_146); +lean_ctor_set(x_190, 2, x_147); +lean_ctor_set(x_190, 3, x_148); +lean_ctor_set(x_190, 4, x_149); +x_191 = lean_st_ref_set(x_8, x_190, x_145); +x_192 = lean_ctor_get(x_191, 1); +lean_inc(x_192); +lean_dec(x_191); +x_193 = lean_box(0); +x_194 = lean_box(x_7); +x_195 = lean_apply_4(x_10, x_193, x_194, x_8, x_192); +return x_195; +} } else { -lean_object* x_157; lean_object* x_158; uint8_t x_159; uint8_t x_160; -x_157 = lean_ctor_get(x_154, 0); -lean_inc(x_157); -lean_dec(x_154); -x_158 = lean_ctor_get(x_43, 0); -lean_inc(x_158); -x_159 = 0; -x_160 = l_String_Range_contains(x_1, x_158, x_159); -lean_dec(x_158); -if (x_160 == 0) +lean_object* x_196; lean_object* x_197; lean_object* x_198; uint64_t x_199; uint64_t x_200; uint64_t x_201; uint64_t x_202; uint64_t x_203; uint64_t x_204; uint64_t x_205; size_t x_206; size_t x_207; size_t x_208; size_t x_209; size_t x_210; lean_object* x_211; uint8_t x_212; +x_196 = lean_ctor_get(x_144, 0); +x_197 = lean_ctor_get(x_144, 1); +lean_inc(x_197); +lean_inc(x_196); +lean_dec(x_144); +x_198 = lean_array_get_size(x_197); +x_199 = l___private_Lean_Syntax_0__String_hashRange____x40_Lean_Syntax___hyg_169_(x_139); +x_200 = 32; +x_201 = lean_uint64_shift_right(x_199, x_200); +x_202 = lean_uint64_xor(x_199, x_201); +x_203 = 16; +x_204 = lean_uint64_shift_right(x_202, x_203); +x_205 = lean_uint64_xor(x_202, x_204); +x_206 = lean_uint64_to_usize(x_205); +x_207 = lean_usize_of_nat(x_198); +lean_dec(x_198); +x_208 = 1; +x_209 = lean_usize_sub(x_207, x_208); +x_210 = lean_usize_land(x_206, x_209); +x_211 = lean_array_uget(x_197, x_210); +x_212 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__7(x_139, x_211); +if (x_212 == 0) +{ +lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; uint8_t x_223; +x_213 = lean_unsigned_to_nat(1u); +x_214 = lean_nat_add(x_196, x_213); +lean_dec(x_196); +x_215 = lean_box(0); +x_216 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_216, 0, x_139); +lean_ctor_set(x_216, 1, x_215); +lean_ctor_set(x_216, 2, x_211); +x_217 = lean_array_uset(x_197, x_210, x_216); +x_218 = lean_unsigned_to_nat(4u); +x_219 = lean_nat_mul(x_214, x_218); +x_220 = lean_unsigned_to_nat(3u); +x_221 = lean_nat_div(x_219, x_220); +lean_dec(x_219); +x_222 = lean_array_get_size(x_217); +x_223 = lean_nat_dec_le(x_221, x_222); +lean_dec(x_222); +lean_dec(x_221); +if (x_223 == 0) { -lean_object* x_161; lean_object* x_162; -lean_dec(x_157); -lean_dec(x_44); -lean_dec(x_43); -lean_dec(x_39); -lean_dec(x_2); -x_161 = lean_box(0); -x_162 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_162, 0, x_161); -lean_ctor_set(x_162, 1, x_6); -return x_162; +lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; +x_224 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__8(x_217); +x_225 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_225, 0, x_214); +lean_ctor_set(x_225, 1, x_224); +x_226 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_226, 0, x_225); +lean_ctor_set(x_226, 1, x_146); +lean_ctor_set(x_226, 2, x_147); +lean_ctor_set(x_226, 3, x_148); +lean_ctor_set(x_226, 4, x_149); +x_227 = lean_st_ref_set(x_8, x_226, x_145); +x_228 = lean_ctor_get(x_227, 1); +lean_inc(x_228); +lean_dec(x_227); +x_229 = lean_box(x_7); +x_230 = lean_apply_4(x_10, x_215, x_229, x_8, x_228); +return x_230; } else { -lean_object* x_163; uint8_t x_164; -x_163 = l_Lean_LocalDecl_userName(x_157); -x_164 = l_Lean_Name_hasMacroScopes(x_163); -lean_dec(x_163); -if (x_164 == 0) -{ -lean_object* x_165; lean_object* x_166; -x_165 = lean_box(0); -x_166 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__3(x_2, x_44, x_43, x_157, x_39, x_165, x_5, x_6); -lean_dec(x_157); -return x_166; +lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; +x_231 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_231, 0, x_214); +lean_ctor_set(x_231, 1, x_217); +x_232 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_232, 0, x_231); +lean_ctor_set(x_232, 1, x_146); +lean_ctor_set(x_232, 2, x_147); +lean_ctor_set(x_232, 3, x_148); +lean_ctor_set(x_232, 4, x_149); +x_233 = lean_st_ref_set(x_8, x_232, x_145); +x_234 = lean_ctor_get(x_233, 1); +lean_inc(x_234); +lean_dec(x_233); +x_235 = lean_box(x_7); +x_236 = lean_apply_4(x_10, x_215, x_235, x_8, x_234); +return x_236; +} } else { -lean_object* x_167; lean_object* x_168; -lean_dec(x_157); -lean_dec(x_44); -lean_dec(x_43); -lean_dec(x_39); -lean_dec(x_2); -x_167 = lean_box(0); -x_168 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_168, 0, x_167); -lean_ctor_set(x_168, 1, x_6); -return x_168; +lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; +lean_dec(x_211); +lean_dec(x_139); +x_237 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_237, 0, x_196); +lean_ctor_set(x_237, 1, x_197); +x_238 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_238, 0, x_237); +lean_ctor_set(x_238, 1, x_146); +lean_ctor_set(x_238, 2, x_147); +lean_ctor_set(x_238, 3, x_148); +lean_ctor_set(x_238, 4, x_149); +x_239 = lean_st_ref_set(x_8, x_238, x_145); +x_240 = lean_ctor_get(x_239, 1); +lean_inc(x_240); +lean_dec(x_239); +x_241 = lean_box(0); +x_242 = lean_box(x_7); +x_243 = lean_apply_4(x_10, x_241, x_242, x_8, x_240); +return x_243; +} +} +} +else +{ +uint8_t x_244; lean_object* x_245; lean_object* x_246; +lean_dec(x_141); +lean_dec(x_139); +lean_dec(x_8); +x_244 = 1; +x_245 = lean_box(x_244); +x_246 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_246, 0, x_245); +lean_ctor_set(x_246, 1, x_9); +return x_246; +} +} +} +} +default: +{ +lean_object* x_247; lean_object* x_248; lean_object* x_249; +lean_dec(x_11); +lean_dec(x_4); +lean_dec(x_1); +x_247 = lean_box(0); +x_248 = lean_box(x_7); +x_249 = lean_apply_4(x_10, x_247, x_248, x_8, x_9); +return x_249; } } } } +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__8(uint8_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, uint8_t x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +if (x_1 == 0) +{ +lean_object* x_10; lean_object* x_11; +x_10 = lean_box(0); +x_11 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__7(x_2, x_3, x_1, x_4, x_5, x_10, x_7, x_8, x_9); +return x_11; } else { -lean_object* x_169; lean_object* x_170; -lean_dec(x_45); -lean_dec(x_44); -lean_dec(x_43); -lean_dec(x_39); -lean_dec(x_37); +uint8_t x_12; lean_object* x_13; lean_object* x_14; +lean_dec(x_8); +lean_dec(x_4); lean_dec(x_2); -x_169 = lean_box(0); -x_170 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_170, 0, x_169); -lean_ctor_set(x_170, 1, x_6); -return x_170; +x_12 = 1; +x_13 = lean_box(x_12); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_13); +lean_ctor_set(x_14, 1, x_9); +return x_14; } } } -case 4: +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__9(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5) { +_start: { -uint8_t x_171; -lean_dec(x_38); -lean_dec(x_2); -x_171 = lean_ctor_get_uint8(x_37, sizeof(void*)*4); -lean_dec(x_37); -if (x_171 == 0) +lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; +x_6 = lean_st_ref_take(x_4, x_5); +x_7 = lean_ctor_get(x_6, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_6, 1); +lean_inc(x_8); +lean_dec(x_6); +x_9 = !lean_is_exclusive(x_7); +if (x_9 == 0) { -lean_object* x_172; lean_object* x_173; -lean_dec(x_3); -x_172 = lean_box(0); -x_173 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_173, 0, x_172); -lean_ctor_set(x_173, 1, x_6); -return x_173; -} -else +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_10 = lean_ctor_get(x_7, 3); +x_11 = lean_ctor_get(x_1, 2); +lean_inc(x_11); +x_12 = l_Lean_Linter_UnusedVariables_followAliases(x_10, x_11); +x_13 = lean_ctor_get(x_1, 1); +lean_inc(x_13); +lean_dec(x_1); +x_14 = !lean_is_exclusive(x_10); +if (x_14 == 0) { -lean_object* x_174; -x_174 = l_Lean_Elab_Info_range_x3f(x_3); -if (lean_obj_tag(x_174) == 0) +lean_object* x_15; lean_object* x_16; lean_object* x_17; uint64_t x_18; uint64_t x_19; uint64_t x_20; uint64_t x_21; uint64_t x_22; uint64_t x_23; uint64_t x_24; size_t x_25; size_t x_26; size_t x_27; size_t x_28; size_t x_29; lean_object* x_30; uint8_t x_31; +x_15 = lean_ctor_get(x_10, 0); +x_16 = lean_ctor_get(x_10, 1); +x_17 = lean_array_get_size(x_16); +x_18 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_13); +x_19 = 32; +x_20 = lean_uint64_shift_right(x_18, x_19); +x_21 = lean_uint64_xor(x_18, x_20); +x_22 = 16; +x_23 = lean_uint64_shift_right(x_21, x_22); +x_24 = lean_uint64_xor(x_21, x_23); +x_25 = lean_uint64_to_usize(x_24); +x_26 = lean_usize_of_nat(x_17); +lean_dec(x_17); +x_27 = 1; +x_28 = lean_usize_sub(x_26, x_27); +x_29 = lean_usize_land(x_25, x_28); +x_30 = lean_array_uget(x_16, x_29); +x_31 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__15(x_13, x_30); +if (x_31 == 0) { -lean_object* x_175; lean_object* x_176; -lean_dec(x_3); -x_175 = lean_box(0); -x_176 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_176, 0, x_175); -lean_ctor_set(x_176, 1, x_6); -return x_176; -} -else +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; +x_32 = lean_unsigned_to_nat(1u); +x_33 = lean_nat_add(x_15, x_32); +lean_dec(x_15); +x_34 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_34, 0, x_13); +lean_ctor_set(x_34, 1, x_12); +lean_ctor_set(x_34, 2, x_30); +x_35 = lean_array_uset(x_16, x_29, x_34); +x_36 = lean_unsigned_to_nat(4u); +x_37 = lean_nat_mul(x_33, x_36); +x_38 = lean_unsigned_to_nat(3u); +x_39 = lean_nat_div(x_37, x_38); +lean_dec(x_37); +x_40 = lean_array_get_size(x_35); +x_41 = lean_nat_dec_le(x_39, x_40); +lean_dec(x_40); +lean_dec(x_39); +if (x_41 == 0) { -lean_object* x_177; lean_object* x_178; lean_object* x_179; -x_177 = lean_ctor_get(x_174, 0); -lean_inc(x_177); -lean_dec(x_174); -x_178 = l_Lean_Elab_Info_stx(x_3); -lean_dec(x_3); -x_179 = l_Lean_Syntax_getHeadInfo(x_178); -lean_dec(x_178); -if (lean_obj_tag(x_179) == 0) -{ -lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; uint8_t x_188; -lean_dec(x_179); -x_180 = lean_st_ref_take(x_5, x_6); -x_181 = lean_ctor_get(x_180, 0); -lean_inc(x_181); -x_182 = lean_ctor_get(x_181, 0); -lean_inc(x_182); -x_183 = lean_ctor_get(x_180, 1); -lean_inc(x_183); -lean_dec(x_180); -x_184 = lean_ctor_get(x_181, 1); -lean_inc(x_184); -x_185 = lean_ctor_get(x_181, 2); -lean_inc(x_185); -x_186 = lean_ctor_get(x_181, 3); -lean_inc(x_186); -x_187 = lean_ctor_get(x_181, 4); -lean_inc(x_187); -lean_dec(x_181); -x_188 = !lean_is_exclusive(x_182); -if (x_188 == 0) -{ -lean_object* x_189; lean_object* x_190; lean_object* x_191; uint64_t x_192; uint64_t x_193; uint64_t x_194; uint64_t x_195; uint64_t x_196; uint64_t x_197; uint64_t x_198; size_t x_199; size_t x_200; size_t x_201; size_t x_202; size_t x_203; lean_object* x_204; uint8_t x_205; -x_189 = lean_ctor_get(x_182, 0); -x_190 = lean_ctor_get(x_182, 1); -x_191 = lean_array_get_size(x_190); -x_192 = l___private_Lean_Syntax_0__String_hashRange____x40_Lean_Syntax___hyg_169_(x_177); -x_193 = 32; -x_194 = lean_uint64_shift_right(x_192, x_193); -x_195 = lean_uint64_xor(x_192, x_194); -x_196 = 16; -x_197 = lean_uint64_shift_right(x_195, x_196); -x_198 = lean_uint64_xor(x_195, x_197); -x_199 = lean_uint64_to_usize(x_198); -x_200 = lean_usize_of_nat(x_191); -lean_dec(x_191); -x_201 = 1; -x_202 = lean_usize_sub(x_200, x_201); -x_203 = lean_usize_land(x_199, x_202); -x_204 = lean_array_uget(x_190, x_203); -x_205 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__7(x_177, x_204); -if (x_205 == 0) -{ -lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; uint8_t x_216; -x_206 = lean_unsigned_to_nat(1u); -x_207 = lean_nat_add(x_189, x_206); -lean_dec(x_189); -x_208 = lean_box(0); -x_209 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_209, 0, x_177); -lean_ctor_set(x_209, 1, x_208); -lean_ctor_set(x_209, 2, x_204); -x_210 = lean_array_uset(x_190, x_203, x_209); -x_211 = lean_unsigned_to_nat(4u); -x_212 = lean_nat_mul(x_207, x_211); -x_213 = lean_unsigned_to_nat(3u); -x_214 = lean_nat_div(x_212, x_213); -lean_dec(x_212); -x_215 = lean_array_get_size(x_210); -x_216 = lean_nat_dec_le(x_214, x_215); -lean_dec(x_215); -lean_dec(x_214); -if (x_216 == 0) +lean_object* x_42; lean_object* x_43; uint8_t x_44; +x_42 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__16(x_35); +lean_ctor_set(x_10, 1, x_42); +lean_ctor_set(x_10, 0, x_33); +x_43 = lean_st_ref_set(x_4, x_7, x_8); +x_44 = !lean_is_exclusive(x_43); +if (x_44 == 0) { -lean_object* x_217; lean_object* x_218; lean_object* x_219; uint8_t x_220; -x_217 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__8(x_210); -lean_ctor_set(x_182, 1, x_217); -lean_ctor_set(x_182, 0, x_207); -x_218 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_218, 0, x_182); -lean_ctor_set(x_218, 1, x_184); -lean_ctor_set(x_218, 2, x_185); -lean_ctor_set(x_218, 3, x_186); -lean_ctor_set(x_218, 4, x_187); -x_219 = lean_st_ref_set(x_5, x_218, x_183); -x_220 = !lean_is_exclusive(x_219); -if (x_220 == 0) -{ -lean_object* x_221; -x_221 = lean_ctor_get(x_219, 0); -lean_dec(x_221); -lean_ctor_set(x_219, 0, x_208); -return x_219; +lean_object* x_45; uint8_t x_46; lean_object* x_47; +x_45 = lean_ctor_get(x_43, 0); +lean_dec(x_45); +x_46 = 1; +x_47 = lean_box(x_46); +lean_ctor_set(x_43, 0, x_47); +return x_43; } else { -lean_object* x_222; lean_object* x_223; -x_222 = lean_ctor_get(x_219, 1); -lean_inc(x_222); -lean_dec(x_219); -x_223 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_223, 0, x_208); -lean_ctor_set(x_223, 1, x_222); -return x_223; +lean_object* x_48; uint8_t x_49; lean_object* x_50; lean_object* x_51; +x_48 = lean_ctor_get(x_43, 1); +lean_inc(x_48); +lean_dec(x_43); +x_49 = 1; +x_50 = lean_box(x_49); +x_51 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_51, 0, x_50); +lean_ctor_set(x_51, 1, x_48); +return x_51; } } else { -lean_object* x_224; lean_object* x_225; uint8_t x_226; -lean_ctor_set(x_182, 1, x_210); -lean_ctor_set(x_182, 0, x_207); -x_224 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_224, 0, x_182); -lean_ctor_set(x_224, 1, x_184); -lean_ctor_set(x_224, 2, x_185); -lean_ctor_set(x_224, 3, x_186); -lean_ctor_set(x_224, 4, x_187); -x_225 = lean_st_ref_set(x_5, x_224, x_183); -x_226 = !lean_is_exclusive(x_225); -if (x_226 == 0) +lean_object* x_52; uint8_t x_53; +lean_ctor_set(x_10, 1, x_35); +lean_ctor_set(x_10, 0, x_33); +x_52 = lean_st_ref_set(x_4, x_7, x_8); +x_53 = !lean_is_exclusive(x_52); +if (x_53 == 0) { -lean_object* x_227; -x_227 = lean_ctor_get(x_225, 0); -lean_dec(x_227); -lean_ctor_set(x_225, 0, x_208); -return x_225; +lean_object* x_54; uint8_t x_55; lean_object* x_56; +x_54 = lean_ctor_get(x_52, 0); +lean_dec(x_54); +x_55 = 1; +x_56 = lean_box(x_55); +lean_ctor_set(x_52, 0, x_56); +return x_52; } else { -lean_object* x_228; lean_object* x_229; -x_228 = lean_ctor_get(x_225, 1); -lean_inc(x_228); -lean_dec(x_225); -x_229 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_229, 0, x_208); -lean_ctor_set(x_229, 1, x_228); -return x_229; +lean_object* x_57; uint8_t x_58; lean_object* x_59; lean_object* x_60; +x_57 = lean_ctor_get(x_52, 1); +lean_inc(x_57); +lean_dec(x_52); +x_58 = 1; +x_59 = lean_box(x_58); +x_60 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_60, 0, x_59); +lean_ctor_set(x_60, 1, x_57); +return x_60; } } } else { -lean_object* x_230; lean_object* x_231; uint8_t x_232; -lean_dec(x_204); -lean_dec(x_177); -x_230 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_230, 0, x_182); -lean_ctor_set(x_230, 1, x_184); -lean_ctor_set(x_230, 2, x_185); -lean_ctor_set(x_230, 3, x_186); -lean_ctor_set(x_230, 4, x_187); -x_231 = lean_st_ref_set(x_5, x_230, x_183); -x_232 = !lean_is_exclusive(x_231); -if (x_232 == 0) -{ -lean_object* x_233; lean_object* x_234; -x_233 = lean_ctor_get(x_231, 0); -lean_dec(x_233); -x_234 = lean_box(0); -lean_ctor_set(x_231, 0, x_234); -return x_231; +lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; uint8_t x_66; +x_61 = lean_box(0); +x_62 = lean_array_uset(x_16, x_29, x_61); +x_63 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__19(x_13, x_12, x_30); +x_64 = lean_array_uset(x_62, x_29, x_63); +lean_ctor_set(x_10, 1, x_64); +x_65 = lean_st_ref_set(x_4, x_7, x_8); +x_66 = !lean_is_exclusive(x_65); +if (x_66 == 0) +{ +lean_object* x_67; uint8_t x_68; lean_object* x_69; +x_67 = lean_ctor_get(x_65, 0); +lean_dec(x_67); +x_68 = 1; +x_69 = lean_box(x_68); +lean_ctor_set(x_65, 0, x_69); +return x_65; } else { -lean_object* x_235; lean_object* x_236; lean_object* x_237; -x_235 = lean_ctor_get(x_231, 1); -lean_inc(x_235); -lean_dec(x_231); -x_236 = lean_box(0); -x_237 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_237, 0, x_236); -lean_ctor_set(x_237, 1, x_235); -return x_237; +lean_object* x_70; uint8_t x_71; lean_object* x_72; lean_object* x_73; +x_70 = lean_ctor_get(x_65, 1); +lean_inc(x_70); +lean_dec(x_65); +x_71 = 1; +x_72 = lean_box(x_71); +x_73 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_73, 0, x_72); +lean_ctor_set(x_73, 1, x_70); +return x_73; } } } else { -lean_object* x_238; lean_object* x_239; lean_object* x_240; uint64_t x_241; uint64_t x_242; uint64_t x_243; uint64_t x_244; uint64_t x_245; uint64_t x_246; uint64_t x_247; size_t x_248; size_t x_249; size_t x_250; size_t x_251; size_t x_252; lean_object* x_253; uint8_t x_254; -x_238 = lean_ctor_get(x_182, 0); -x_239 = lean_ctor_get(x_182, 1); -lean_inc(x_239); -lean_inc(x_238); -lean_dec(x_182); -x_240 = lean_array_get_size(x_239); -x_241 = l___private_Lean_Syntax_0__String_hashRange____x40_Lean_Syntax___hyg_169_(x_177); -x_242 = 32; -x_243 = lean_uint64_shift_right(x_241, x_242); -x_244 = lean_uint64_xor(x_241, x_243); -x_245 = 16; -x_246 = lean_uint64_shift_right(x_244, x_245); -x_247 = lean_uint64_xor(x_244, x_246); -x_248 = lean_uint64_to_usize(x_247); -x_249 = lean_usize_of_nat(x_240); -lean_dec(x_240); -x_250 = 1; -x_251 = lean_usize_sub(x_249, x_250); -x_252 = lean_usize_land(x_248, x_251); -x_253 = lean_array_uget(x_239, x_252); -x_254 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__7(x_177, x_253); -if (x_254 == 0) -{ -lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; uint8_t x_265; -x_255 = lean_unsigned_to_nat(1u); -x_256 = lean_nat_add(x_238, x_255); -lean_dec(x_238); -x_257 = lean_box(0); -x_258 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_258, 0, x_177); -lean_ctor_set(x_258, 1, x_257); -lean_ctor_set(x_258, 2, x_253); -x_259 = lean_array_uset(x_239, x_252, x_258); -x_260 = lean_unsigned_to_nat(4u); -x_261 = lean_nat_mul(x_256, x_260); -x_262 = lean_unsigned_to_nat(3u); -x_263 = lean_nat_div(x_261, x_262); -lean_dec(x_261); -x_264 = lean_array_get_size(x_259); -x_265 = lean_nat_dec_le(x_263, x_264); -lean_dec(x_264); -lean_dec(x_263); -if (x_265 == 0) -{ -lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; -x_266 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__8(x_259); -x_267 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_267, 0, x_256); -lean_ctor_set(x_267, 1, x_266); -x_268 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_268, 0, x_267); -lean_ctor_set(x_268, 1, x_184); -lean_ctor_set(x_268, 2, x_185); -lean_ctor_set(x_268, 3, x_186); -lean_ctor_set(x_268, 4, x_187); -x_269 = lean_st_ref_set(x_5, x_268, x_183); -x_270 = lean_ctor_get(x_269, 1); -lean_inc(x_270); -if (lean_is_exclusive(x_269)) { - lean_ctor_release(x_269, 0); - lean_ctor_release(x_269, 1); - x_271 = x_269; +lean_object* x_74; lean_object* x_75; lean_object* x_76; uint64_t x_77; uint64_t x_78; uint64_t x_79; uint64_t x_80; uint64_t x_81; uint64_t x_82; uint64_t x_83; size_t x_84; size_t x_85; size_t x_86; size_t x_87; size_t x_88; lean_object* x_89; uint8_t x_90; +x_74 = lean_ctor_get(x_10, 0); +x_75 = lean_ctor_get(x_10, 1); +lean_inc(x_75); +lean_inc(x_74); +lean_dec(x_10); +x_76 = lean_array_get_size(x_75); +x_77 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_13); +x_78 = 32; +x_79 = lean_uint64_shift_right(x_77, x_78); +x_80 = lean_uint64_xor(x_77, x_79); +x_81 = 16; +x_82 = lean_uint64_shift_right(x_80, x_81); +x_83 = lean_uint64_xor(x_80, x_82); +x_84 = lean_uint64_to_usize(x_83); +x_85 = lean_usize_of_nat(x_76); +lean_dec(x_76); +x_86 = 1; +x_87 = lean_usize_sub(x_85, x_86); +x_88 = lean_usize_land(x_84, x_87); +x_89 = lean_array_uget(x_75, x_88); +x_90 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__15(x_13, x_89); +if (x_90 == 0) +{ +lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; uint8_t x_100; +x_91 = lean_unsigned_to_nat(1u); +x_92 = lean_nat_add(x_74, x_91); +lean_dec(x_74); +x_93 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_93, 0, x_13); +lean_ctor_set(x_93, 1, x_12); +lean_ctor_set(x_93, 2, x_89); +x_94 = lean_array_uset(x_75, x_88, x_93); +x_95 = lean_unsigned_to_nat(4u); +x_96 = lean_nat_mul(x_92, x_95); +x_97 = lean_unsigned_to_nat(3u); +x_98 = lean_nat_div(x_96, x_97); +lean_dec(x_96); +x_99 = lean_array_get_size(x_94); +x_100 = lean_nat_dec_le(x_98, x_99); +lean_dec(x_99); +lean_dec(x_98); +if (x_100 == 0) +{ +lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; uint8_t x_106; lean_object* x_107; lean_object* x_108; +x_101 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__16(x_94); +x_102 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_102, 0, x_92); +lean_ctor_set(x_102, 1, x_101); +lean_ctor_set(x_7, 3, x_102); +x_103 = lean_st_ref_set(x_4, x_7, x_8); +x_104 = lean_ctor_get(x_103, 1); +lean_inc(x_104); +if (lean_is_exclusive(x_103)) { + lean_ctor_release(x_103, 0); + lean_ctor_release(x_103, 1); + x_105 = x_103; } else { - lean_dec_ref(x_269); - x_271 = lean_box(0); + lean_dec_ref(x_103); + x_105 = lean_box(0); } -if (lean_is_scalar(x_271)) { - x_272 = lean_alloc_ctor(0, 2, 0); +x_106 = 1; +x_107 = lean_box(x_106); +if (lean_is_scalar(x_105)) { + x_108 = lean_alloc_ctor(0, 2, 0); } else { - x_272 = x_271; -} -lean_ctor_set(x_272, 0, x_257); -lean_ctor_set(x_272, 1, x_270); -return x_272; -} -else -{ -lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; -x_273 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_273, 0, x_256); -lean_ctor_set(x_273, 1, x_259); -x_274 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_274, 0, x_273); -lean_ctor_set(x_274, 1, x_184); -lean_ctor_set(x_274, 2, x_185); -lean_ctor_set(x_274, 3, x_186); -lean_ctor_set(x_274, 4, x_187); -x_275 = lean_st_ref_set(x_5, x_274, x_183); -x_276 = lean_ctor_get(x_275, 1); -lean_inc(x_276); -if (lean_is_exclusive(x_275)) { - lean_ctor_release(x_275, 0); - lean_ctor_release(x_275, 1); - x_277 = x_275; + x_108 = x_105; +} +lean_ctor_set(x_108, 0, x_107); +lean_ctor_set(x_108, 1, x_104); +return x_108; +} +else +{ +lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; uint8_t x_113; lean_object* x_114; lean_object* x_115; +x_109 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_109, 0, x_92); +lean_ctor_set(x_109, 1, x_94); +lean_ctor_set(x_7, 3, x_109); +x_110 = lean_st_ref_set(x_4, x_7, x_8); +x_111 = lean_ctor_get(x_110, 1); +lean_inc(x_111); +if (lean_is_exclusive(x_110)) { + lean_ctor_release(x_110, 0); + lean_ctor_release(x_110, 1); + x_112 = x_110; } else { - lean_dec_ref(x_275); - x_277 = lean_box(0); + lean_dec_ref(x_110); + x_112 = lean_box(0); } -if (lean_is_scalar(x_277)) { - x_278 = lean_alloc_ctor(0, 2, 0); +x_113 = 1; +x_114 = lean_box(x_113); +if (lean_is_scalar(x_112)) { + x_115 = lean_alloc_ctor(0, 2, 0); } else { - x_278 = x_277; + x_115 = x_112; } -lean_ctor_set(x_278, 0, x_257); -lean_ctor_set(x_278, 1, x_276); -return x_278; +lean_ctor_set(x_115, 0, x_114); +lean_ctor_set(x_115, 1, x_111); +return x_115; } } else { -lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; -lean_dec(x_253); -lean_dec(x_177); -x_279 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_279, 0, x_238); -lean_ctor_set(x_279, 1, x_239); -x_280 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_280, 0, x_279); -lean_ctor_set(x_280, 1, x_184); -lean_ctor_set(x_280, 2, x_185); -lean_ctor_set(x_280, 3, x_186); -lean_ctor_set(x_280, 4, x_187); -x_281 = lean_st_ref_set(x_5, x_280, x_183); -x_282 = lean_ctor_get(x_281, 1); -lean_inc(x_282); -if (lean_is_exclusive(x_281)) { - lean_ctor_release(x_281, 0); - lean_ctor_release(x_281, 1); - x_283 = x_281; +lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; uint8_t x_124; lean_object* x_125; lean_object* x_126; +x_116 = lean_box(0); +x_117 = lean_array_uset(x_75, x_88, x_116); +x_118 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__19(x_13, x_12, x_89); +x_119 = lean_array_uset(x_117, x_88, x_118); +x_120 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_120, 0, x_74); +lean_ctor_set(x_120, 1, x_119); +lean_ctor_set(x_7, 3, x_120); +x_121 = lean_st_ref_set(x_4, x_7, x_8); +x_122 = lean_ctor_get(x_121, 1); +lean_inc(x_122); +if (lean_is_exclusive(x_121)) { + lean_ctor_release(x_121, 0); + lean_ctor_release(x_121, 1); + x_123 = x_121; } else { - lean_dec_ref(x_281); - x_283 = lean_box(0); + lean_dec_ref(x_121); + x_123 = lean_box(0); } -x_284 = lean_box(0); -if (lean_is_scalar(x_283)) { - x_285 = lean_alloc_ctor(0, 2, 0); +x_124 = 1; +x_125 = lean_box(x_124); +if (lean_is_scalar(x_123)) { + x_126 = lean_alloc_ctor(0, 2, 0); } else { - x_285 = x_283; -} -lean_ctor_set(x_285, 0, x_284); -lean_ctor_set(x_285, 1, x_282); -return x_285; -} -} -} -else -{ -lean_object* x_286; lean_object* x_287; -lean_dec(x_179); -lean_dec(x_177); -x_286 = lean_box(0); -x_287 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_287, 0, x_286); -lean_ctor_set(x_287, 1, x_6); -return x_287; -} -} -} -} -default: -{ -lean_object* x_288; lean_object* x_289; -lean_dec(x_38); -lean_dec(x_37); -lean_dec(x_3); -lean_dec(x_2); -x_288 = lean_box(0); -x_289 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_289, 0, x_288); -lean_ctor_set(x_289, 1, x_6); -return x_289; -} -} -} -case 9: -{ -lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; uint8_t x_294; -lean_dec(x_2); -x_290 = lean_ctor_get(x_3, 0); -lean_inc(x_290); -lean_dec(x_3); -x_291 = lean_st_ref_take(x_5, x_6); -x_292 = lean_ctor_get(x_291, 0); -lean_inc(x_292); -x_293 = lean_ctor_get(x_291, 1); -lean_inc(x_293); -lean_dec(x_291); -x_294 = !lean_is_exclusive(x_292); -if (x_294 == 0) -{ -lean_object* x_295; lean_object* x_296; lean_object* x_297; lean_object* x_298; uint8_t x_299; -x_295 = lean_ctor_get(x_292, 3); -x_296 = lean_ctor_get(x_290, 2); -lean_inc(x_296); -x_297 = l_Lean_Linter_UnusedVariables_followAliases(x_295, x_296); -x_298 = lean_ctor_get(x_290, 1); -lean_inc(x_298); -lean_dec(x_290); -x_299 = !lean_is_exclusive(x_295); -if (x_299 == 0) -{ -lean_object* x_300; lean_object* x_301; lean_object* x_302; uint64_t x_303; uint64_t x_304; uint64_t x_305; uint64_t x_306; uint64_t x_307; uint64_t x_308; uint64_t x_309; size_t x_310; size_t x_311; size_t x_312; size_t x_313; size_t x_314; lean_object* x_315; uint8_t x_316; -x_300 = lean_ctor_get(x_295, 0); -x_301 = lean_ctor_get(x_295, 1); -x_302 = lean_array_get_size(x_301); -x_303 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_298); -x_304 = 32; -x_305 = lean_uint64_shift_right(x_303, x_304); -x_306 = lean_uint64_xor(x_303, x_305); -x_307 = 16; -x_308 = lean_uint64_shift_right(x_306, x_307); -x_309 = lean_uint64_xor(x_306, x_308); -x_310 = lean_uint64_to_usize(x_309); -x_311 = lean_usize_of_nat(x_302); -lean_dec(x_302); -x_312 = 1; -x_313 = lean_usize_sub(x_311, x_312); -x_314 = lean_usize_land(x_310, x_313); -x_315 = lean_array_uget(x_301, x_314); -x_316 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__11(x_298, x_315); -if (x_316 == 0) -{ -lean_object* x_317; lean_object* x_318; lean_object* x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; lean_object* x_324; lean_object* x_325; uint8_t x_326; -x_317 = lean_unsigned_to_nat(1u); -x_318 = lean_nat_add(x_300, x_317); -lean_dec(x_300); -x_319 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_319, 0, x_298); -lean_ctor_set(x_319, 1, x_297); -lean_ctor_set(x_319, 2, x_315); -x_320 = lean_array_uset(x_301, x_314, x_319); -x_321 = lean_unsigned_to_nat(4u); -x_322 = lean_nat_mul(x_318, x_321); -x_323 = lean_unsigned_to_nat(3u); -x_324 = lean_nat_div(x_322, x_323); -lean_dec(x_322); -x_325 = lean_array_get_size(x_320); -x_326 = lean_nat_dec_le(x_324, x_325); -lean_dec(x_325); -lean_dec(x_324); -if (x_326 == 0) -{ -lean_object* x_327; lean_object* x_328; uint8_t x_329; -x_327 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__12(x_320); -lean_ctor_set(x_295, 1, x_327); -lean_ctor_set(x_295, 0, x_318); -x_328 = lean_st_ref_set(x_5, x_292, x_293); -x_329 = !lean_is_exclusive(x_328); -if (x_329 == 0) -{ -lean_object* x_330; lean_object* x_331; -x_330 = lean_ctor_get(x_328, 0); -lean_dec(x_330); -x_331 = lean_box(0); -lean_ctor_set(x_328, 0, x_331); -return x_328; -} -else -{ -lean_object* x_332; lean_object* x_333; lean_object* x_334; -x_332 = lean_ctor_get(x_328, 1); -lean_inc(x_332); -lean_dec(x_328); -x_333 = lean_box(0); -x_334 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_334, 0, x_333); -lean_ctor_set(x_334, 1, x_332); -return x_334; -} -} -else -{ -lean_object* x_335; uint8_t x_336; -lean_ctor_set(x_295, 1, x_320); -lean_ctor_set(x_295, 0, x_318); -x_335 = lean_st_ref_set(x_5, x_292, x_293); -x_336 = !lean_is_exclusive(x_335); -if (x_336 == 0) -{ -lean_object* x_337; lean_object* x_338; -x_337 = lean_ctor_get(x_335, 0); -lean_dec(x_337); -x_338 = lean_box(0); -lean_ctor_set(x_335, 0, x_338); -return x_335; -} -else -{ -lean_object* x_339; lean_object* x_340; lean_object* x_341; -x_339 = lean_ctor_get(x_335, 1); -lean_inc(x_339); -lean_dec(x_335); -x_340 = lean_box(0); -x_341 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_341, 0, x_340); -lean_ctor_set(x_341, 1, x_339); -return x_341; + x_126 = x_123; } +lean_ctor_set(x_126, 0, x_125); +lean_ctor_set(x_126, 1, x_122); +return x_126; } } -else -{ -lean_object* x_342; lean_object* x_343; lean_object* x_344; lean_object* x_345; lean_object* x_346; uint8_t x_347; -x_342 = lean_box(0); -x_343 = lean_array_uset(x_301, x_314, x_342); -x_344 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__15(x_298, x_297, x_315); -x_345 = lean_array_uset(x_343, x_314, x_344); -lean_ctor_set(x_295, 1, x_345); -x_346 = lean_st_ref_set(x_5, x_292, x_293); -x_347 = !lean_is_exclusive(x_346); -if (x_347 == 0) -{ -lean_object* x_348; lean_object* x_349; -x_348 = lean_ctor_get(x_346, 0); -lean_dec(x_348); -x_349 = lean_box(0); -lean_ctor_set(x_346, 0, x_349); -return x_346; } else { -lean_object* x_350; lean_object* x_351; lean_object* x_352; -x_350 = lean_ctor_get(x_346, 1); -lean_inc(x_350); -lean_dec(x_346); -x_351 = lean_box(0); -x_352 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_352, 0, x_351); -lean_ctor_set(x_352, 1, x_350); -return x_352; -} -} -} -else -{ -lean_object* x_353; lean_object* x_354; lean_object* x_355; uint64_t x_356; uint64_t x_357; uint64_t x_358; uint64_t x_359; uint64_t x_360; uint64_t x_361; uint64_t x_362; size_t x_363; size_t x_364; size_t x_365; size_t x_366; size_t x_367; lean_object* x_368; uint8_t x_369; -x_353 = lean_ctor_get(x_295, 0); -x_354 = lean_ctor_get(x_295, 1); -lean_inc(x_354); -lean_inc(x_353); -lean_dec(x_295); -x_355 = lean_array_get_size(x_354); -x_356 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_298); -x_357 = 32; -x_358 = lean_uint64_shift_right(x_356, x_357); -x_359 = lean_uint64_xor(x_356, x_358); -x_360 = 16; -x_361 = lean_uint64_shift_right(x_359, x_360); -x_362 = lean_uint64_xor(x_359, x_361); -x_363 = lean_uint64_to_usize(x_362); -x_364 = lean_usize_of_nat(x_355); -lean_dec(x_355); -x_365 = 1; -x_366 = lean_usize_sub(x_364, x_365); -x_367 = lean_usize_land(x_363, x_366); -x_368 = lean_array_uget(x_354, x_367); -x_369 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__11(x_298, x_368); -if (x_369 == 0) -{ -lean_object* x_370; lean_object* x_371; lean_object* x_372; lean_object* x_373; lean_object* x_374; lean_object* x_375; lean_object* x_376; lean_object* x_377; lean_object* x_378; uint8_t x_379; -x_370 = lean_unsigned_to_nat(1u); -x_371 = lean_nat_add(x_353, x_370); -lean_dec(x_353); -x_372 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_372, 0, x_298); -lean_ctor_set(x_372, 1, x_297); -lean_ctor_set(x_372, 2, x_368); -x_373 = lean_array_uset(x_354, x_367, x_372); -x_374 = lean_unsigned_to_nat(4u); -x_375 = lean_nat_mul(x_371, x_374); -x_376 = lean_unsigned_to_nat(3u); -x_377 = lean_nat_div(x_375, x_376); -lean_dec(x_375); -x_378 = lean_array_get_size(x_373); -x_379 = lean_nat_dec_le(x_377, x_378); -lean_dec(x_378); -lean_dec(x_377); -if (x_379 == 0) -{ -lean_object* x_380; lean_object* x_381; lean_object* x_382; lean_object* x_383; lean_object* x_384; lean_object* x_385; lean_object* x_386; -x_380 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__12(x_373); -x_381 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_381, 0, x_371); -lean_ctor_set(x_381, 1, x_380); -lean_ctor_set(x_292, 3, x_381); -x_382 = lean_st_ref_set(x_5, x_292, x_293); -x_383 = lean_ctor_get(x_382, 1); -lean_inc(x_383); -if (lean_is_exclusive(x_382)) { - lean_ctor_release(x_382, 0); - lean_ctor_release(x_382, 1); - x_384 = x_382; -} else { - lean_dec_ref(x_382); - x_384 = lean_box(0); -} -x_385 = lean_box(0); -if (lean_is_scalar(x_384)) { - x_386 = lean_alloc_ctor(0, 2, 0); -} else { - x_386 = x_384; -} -lean_ctor_set(x_386, 0, x_385); -lean_ctor_set(x_386, 1, x_383); -return x_386; -} -else -{ -lean_object* x_387; lean_object* x_388; lean_object* x_389; lean_object* x_390; lean_object* x_391; lean_object* x_392; -x_387 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_387, 0, x_371); -lean_ctor_set(x_387, 1, x_373); -lean_ctor_set(x_292, 3, x_387); -x_388 = lean_st_ref_set(x_5, x_292, x_293); -x_389 = lean_ctor_get(x_388, 1); -lean_inc(x_389); -if (lean_is_exclusive(x_388)) { - lean_ctor_release(x_388, 0); - lean_ctor_release(x_388, 1); - x_390 = x_388; -} else { - lean_dec_ref(x_388); - x_390 = lean_box(0); -} -x_391 = lean_box(0); -if (lean_is_scalar(x_390)) { - x_392 = lean_alloc_ctor(0, 2, 0); -} else { - x_392 = x_390; -} -lean_ctor_set(x_392, 0, x_391); -lean_ctor_set(x_392, 1, x_389); -return x_392; -} -} -else -{ -lean_object* x_393; lean_object* x_394; lean_object* x_395; lean_object* x_396; lean_object* x_397; lean_object* x_398; lean_object* x_399; lean_object* x_400; lean_object* x_401; lean_object* x_402; -x_393 = lean_box(0); -x_394 = lean_array_uset(x_354, x_367, x_393); -x_395 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__15(x_298, x_297, x_368); -x_396 = lean_array_uset(x_394, x_367, x_395); -x_397 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_397, 0, x_353); -lean_ctor_set(x_397, 1, x_396); -lean_ctor_set(x_292, 3, x_397); -x_398 = lean_st_ref_set(x_5, x_292, x_293); -x_399 = lean_ctor_get(x_398, 1); -lean_inc(x_399); -if (lean_is_exclusive(x_398)) { - lean_ctor_release(x_398, 0); - lean_ctor_release(x_398, 1); - x_400 = x_398; -} else { - lean_dec_ref(x_398); - x_400 = lean_box(0); -} -x_401 = lean_box(0); -if (lean_is_scalar(x_400)) { - x_402 = lean_alloc_ctor(0, 2, 0); -} else { - x_402 = x_400; -} -lean_ctor_set(x_402, 0, x_401); -lean_ctor_set(x_402, 1, x_399); -return x_402; -} -} -} -else -{ -lean_object* x_403; lean_object* x_404; lean_object* x_405; lean_object* x_406; lean_object* x_407; lean_object* x_408; lean_object* x_409; lean_object* x_410; lean_object* x_411; lean_object* x_412; lean_object* x_413; lean_object* x_414; uint64_t x_415; uint64_t x_416; uint64_t x_417; uint64_t x_418; uint64_t x_419; uint64_t x_420; uint64_t x_421; size_t x_422; size_t x_423; size_t x_424; size_t x_425; size_t x_426; lean_object* x_427; uint8_t x_428; -x_403 = lean_ctor_get(x_292, 0); -x_404 = lean_ctor_get(x_292, 1); -x_405 = lean_ctor_get(x_292, 2); -x_406 = lean_ctor_get(x_292, 3); -x_407 = lean_ctor_get(x_292, 4); -lean_inc(x_407); -lean_inc(x_406); -lean_inc(x_405); -lean_inc(x_404); -lean_inc(x_403); -lean_dec(x_292); -x_408 = lean_ctor_get(x_290, 2); -lean_inc(x_408); -x_409 = l_Lean_Linter_UnusedVariables_followAliases(x_406, x_408); -x_410 = lean_ctor_get(x_290, 1); -lean_inc(x_410); -lean_dec(x_290); -x_411 = lean_ctor_get(x_406, 0); -lean_inc(x_411); -x_412 = lean_ctor_get(x_406, 1); -lean_inc(x_412); -if (lean_is_exclusive(x_406)) { - lean_ctor_release(x_406, 0); - lean_ctor_release(x_406, 1); - x_413 = x_406; +lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; uint64_t x_139; uint64_t x_140; uint64_t x_141; uint64_t x_142; uint64_t x_143; uint64_t x_144; uint64_t x_145; size_t x_146; size_t x_147; size_t x_148; size_t x_149; size_t x_150; lean_object* x_151; uint8_t x_152; +x_127 = lean_ctor_get(x_7, 0); +x_128 = lean_ctor_get(x_7, 1); +x_129 = lean_ctor_get(x_7, 2); +x_130 = lean_ctor_get(x_7, 3); +x_131 = lean_ctor_get(x_7, 4); +lean_inc(x_131); +lean_inc(x_130); +lean_inc(x_129); +lean_inc(x_128); +lean_inc(x_127); +lean_dec(x_7); +x_132 = lean_ctor_get(x_1, 2); +lean_inc(x_132); +x_133 = l_Lean_Linter_UnusedVariables_followAliases(x_130, x_132); +x_134 = lean_ctor_get(x_1, 1); +lean_inc(x_134); +lean_dec(x_1); +x_135 = lean_ctor_get(x_130, 0); +lean_inc(x_135); +x_136 = lean_ctor_get(x_130, 1); +lean_inc(x_136); +if (lean_is_exclusive(x_130)) { + lean_ctor_release(x_130, 0); + lean_ctor_release(x_130, 1); + x_137 = x_130; } else { - lean_dec_ref(x_406); - x_413 = lean_box(0); -} -x_414 = lean_array_get_size(x_412); -x_415 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_410); -x_416 = 32; -x_417 = lean_uint64_shift_right(x_415, x_416); -x_418 = lean_uint64_xor(x_415, x_417); -x_419 = 16; -x_420 = lean_uint64_shift_right(x_418, x_419); -x_421 = lean_uint64_xor(x_418, x_420); -x_422 = lean_uint64_to_usize(x_421); -x_423 = lean_usize_of_nat(x_414); -lean_dec(x_414); -x_424 = 1; -x_425 = lean_usize_sub(x_423, x_424); -x_426 = lean_usize_land(x_422, x_425); -x_427 = lean_array_uget(x_412, x_426); -x_428 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__11(x_410, x_427); -if (x_428 == 0) -{ -lean_object* x_429; lean_object* x_430; lean_object* x_431; lean_object* x_432; lean_object* x_433; lean_object* x_434; lean_object* x_435; lean_object* x_436; lean_object* x_437; uint8_t x_438; -x_429 = lean_unsigned_to_nat(1u); -x_430 = lean_nat_add(x_411, x_429); -lean_dec(x_411); -x_431 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_431, 0, x_410); -lean_ctor_set(x_431, 1, x_409); -lean_ctor_set(x_431, 2, x_427); -x_432 = lean_array_uset(x_412, x_426, x_431); -x_433 = lean_unsigned_to_nat(4u); -x_434 = lean_nat_mul(x_430, x_433); -x_435 = lean_unsigned_to_nat(3u); -x_436 = lean_nat_div(x_434, x_435); -lean_dec(x_434); -x_437 = lean_array_get_size(x_432); -x_438 = lean_nat_dec_le(x_436, x_437); -lean_dec(x_437); -lean_dec(x_436); -if (x_438 == 0) -{ -lean_object* x_439; lean_object* x_440; lean_object* x_441; lean_object* x_442; lean_object* x_443; lean_object* x_444; lean_object* x_445; lean_object* x_446; -x_439 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__12(x_432); -if (lean_is_scalar(x_413)) { - x_440 = lean_alloc_ctor(0, 2, 0); + lean_dec_ref(x_130); + x_137 = lean_box(0); +} +x_138 = lean_array_get_size(x_136); +x_139 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_134); +x_140 = 32; +x_141 = lean_uint64_shift_right(x_139, x_140); +x_142 = lean_uint64_xor(x_139, x_141); +x_143 = 16; +x_144 = lean_uint64_shift_right(x_142, x_143); +x_145 = lean_uint64_xor(x_142, x_144); +x_146 = lean_uint64_to_usize(x_145); +x_147 = lean_usize_of_nat(x_138); +lean_dec(x_138); +x_148 = 1; +x_149 = lean_usize_sub(x_147, x_148); +x_150 = lean_usize_land(x_146, x_149); +x_151 = lean_array_uget(x_136, x_150); +x_152 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__15(x_134, x_151); +if (x_152 == 0) +{ +lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; uint8_t x_162; +x_153 = lean_unsigned_to_nat(1u); +x_154 = lean_nat_add(x_135, x_153); +lean_dec(x_135); +x_155 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_155, 0, x_134); +lean_ctor_set(x_155, 1, x_133); +lean_ctor_set(x_155, 2, x_151); +x_156 = lean_array_uset(x_136, x_150, x_155); +x_157 = lean_unsigned_to_nat(4u); +x_158 = lean_nat_mul(x_154, x_157); +x_159 = lean_unsigned_to_nat(3u); +x_160 = lean_nat_div(x_158, x_159); +lean_dec(x_158); +x_161 = lean_array_get_size(x_156); +x_162 = lean_nat_dec_le(x_160, x_161); +lean_dec(x_161); +lean_dec(x_160); +if (x_162 == 0) +{ +lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; uint8_t x_169; lean_object* x_170; lean_object* x_171; +x_163 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__16(x_156); +if (lean_is_scalar(x_137)) { + x_164 = lean_alloc_ctor(0, 2, 0); } else { - x_440 = x_413; -} -lean_ctor_set(x_440, 0, x_430); -lean_ctor_set(x_440, 1, x_439); -x_441 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_441, 0, x_403); -lean_ctor_set(x_441, 1, x_404); -lean_ctor_set(x_441, 2, x_405); -lean_ctor_set(x_441, 3, x_440); -lean_ctor_set(x_441, 4, x_407); -x_442 = lean_st_ref_set(x_5, x_441, x_293); -x_443 = lean_ctor_get(x_442, 1); -lean_inc(x_443); -if (lean_is_exclusive(x_442)) { - lean_ctor_release(x_442, 0); - lean_ctor_release(x_442, 1); - x_444 = x_442; + x_164 = x_137; +} +lean_ctor_set(x_164, 0, x_154); +lean_ctor_set(x_164, 1, x_163); +x_165 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_165, 0, x_127); +lean_ctor_set(x_165, 1, x_128); +lean_ctor_set(x_165, 2, x_129); +lean_ctor_set(x_165, 3, x_164); +lean_ctor_set(x_165, 4, x_131); +x_166 = lean_st_ref_set(x_4, x_165, x_8); +x_167 = lean_ctor_get(x_166, 1); +lean_inc(x_167); +if (lean_is_exclusive(x_166)) { + lean_ctor_release(x_166, 0); + lean_ctor_release(x_166, 1); + x_168 = x_166; } else { - lean_dec_ref(x_442); - x_444 = lean_box(0); + lean_dec_ref(x_166); + x_168 = lean_box(0); } -x_445 = lean_box(0); -if (lean_is_scalar(x_444)) { - x_446 = lean_alloc_ctor(0, 2, 0); +x_169 = 1; +x_170 = lean_box(x_169); +if (lean_is_scalar(x_168)) { + x_171 = lean_alloc_ctor(0, 2, 0); } else { - x_446 = x_444; + x_171 = x_168; } -lean_ctor_set(x_446, 0, x_445); -lean_ctor_set(x_446, 1, x_443); -return x_446; +lean_ctor_set(x_171, 0, x_170); +lean_ctor_set(x_171, 1, x_167); +return x_171; } else { -lean_object* x_447; lean_object* x_448; lean_object* x_449; lean_object* x_450; lean_object* x_451; lean_object* x_452; lean_object* x_453; -if (lean_is_scalar(x_413)) { - x_447 = lean_alloc_ctor(0, 2, 0); +lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; uint8_t x_177; lean_object* x_178; lean_object* x_179; +if (lean_is_scalar(x_137)) { + x_172 = lean_alloc_ctor(0, 2, 0); } else { - x_447 = x_413; -} -lean_ctor_set(x_447, 0, x_430); -lean_ctor_set(x_447, 1, x_432); -x_448 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_448, 0, x_403); -lean_ctor_set(x_448, 1, x_404); -lean_ctor_set(x_448, 2, x_405); -lean_ctor_set(x_448, 3, x_447); -lean_ctor_set(x_448, 4, x_407); -x_449 = lean_st_ref_set(x_5, x_448, x_293); -x_450 = lean_ctor_get(x_449, 1); -lean_inc(x_450); -if (lean_is_exclusive(x_449)) { - lean_ctor_release(x_449, 0); - lean_ctor_release(x_449, 1); - x_451 = x_449; + x_172 = x_137; +} +lean_ctor_set(x_172, 0, x_154); +lean_ctor_set(x_172, 1, x_156); +x_173 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_173, 0, x_127); +lean_ctor_set(x_173, 1, x_128); +lean_ctor_set(x_173, 2, x_129); +lean_ctor_set(x_173, 3, x_172); +lean_ctor_set(x_173, 4, x_131); +x_174 = lean_st_ref_set(x_4, x_173, x_8); +x_175 = lean_ctor_get(x_174, 1); +lean_inc(x_175); +if (lean_is_exclusive(x_174)) { + lean_ctor_release(x_174, 0); + lean_ctor_release(x_174, 1); + x_176 = x_174; } else { - lean_dec_ref(x_449); - x_451 = lean_box(0); + lean_dec_ref(x_174); + x_176 = lean_box(0); } -x_452 = lean_box(0); -if (lean_is_scalar(x_451)) { - x_453 = lean_alloc_ctor(0, 2, 0); +x_177 = 1; +x_178 = lean_box(x_177); +if (lean_is_scalar(x_176)) { + x_179 = lean_alloc_ctor(0, 2, 0); } else { - x_453 = x_451; + x_179 = x_176; } -lean_ctor_set(x_453, 0, x_452); -lean_ctor_set(x_453, 1, x_450); -return x_453; +lean_ctor_set(x_179, 0, x_178); +lean_ctor_set(x_179, 1, x_175); +return x_179; } } else { -lean_object* x_454; lean_object* x_455; lean_object* x_456; lean_object* x_457; lean_object* x_458; lean_object* x_459; lean_object* x_460; lean_object* x_461; lean_object* x_462; lean_object* x_463; lean_object* x_464; -x_454 = lean_box(0); -x_455 = lean_array_uset(x_412, x_426, x_454); -x_456 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__15(x_410, x_409, x_427); -x_457 = lean_array_uset(x_455, x_426, x_456); -if (lean_is_scalar(x_413)) { - x_458 = lean_alloc_ctor(0, 2, 0); +lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; uint8_t x_189; lean_object* x_190; lean_object* x_191; +x_180 = lean_box(0); +x_181 = lean_array_uset(x_136, x_150, x_180); +x_182 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__19(x_134, x_133, x_151); +x_183 = lean_array_uset(x_181, x_150, x_182); +if (lean_is_scalar(x_137)) { + x_184 = lean_alloc_ctor(0, 2, 0); } else { - x_458 = x_413; -} -lean_ctor_set(x_458, 0, x_411); -lean_ctor_set(x_458, 1, x_457); -x_459 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_459, 0, x_403); -lean_ctor_set(x_459, 1, x_404); -lean_ctor_set(x_459, 2, x_405); -lean_ctor_set(x_459, 3, x_458); -lean_ctor_set(x_459, 4, x_407); -x_460 = lean_st_ref_set(x_5, x_459, x_293); -x_461 = lean_ctor_get(x_460, 1); -lean_inc(x_461); -if (lean_is_exclusive(x_460)) { - lean_ctor_release(x_460, 0); - lean_ctor_release(x_460, 1); - x_462 = x_460; + x_184 = x_137; +} +lean_ctor_set(x_184, 0, x_135); +lean_ctor_set(x_184, 1, x_183); +x_185 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_185, 0, x_127); +lean_ctor_set(x_185, 1, x_128); +lean_ctor_set(x_185, 2, x_129); +lean_ctor_set(x_185, 3, x_184); +lean_ctor_set(x_185, 4, x_131); +x_186 = lean_st_ref_set(x_4, x_185, x_8); +x_187 = lean_ctor_get(x_186, 1); +lean_inc(x_187); +if (lean_is_exclusive(x_186)) { + lean_ctor_release(x_186, 0); + lean_ctor_release(x_186, 1); + x_188 = x_186; } else { - lean_dec_ref(x_460); - x_462 = lean_box(0); + lean_dec_ref(x_186); + x_188 = lean_box(0); } -x_463 = lean_box(0); -if (lean_is_scalar(x_462)) { - x_464 = lean_alloc_ctor(0, 2, 0); +x_189 = 1; +x_190 = lean_box(x_189); +if (lean_is_scalar(x_188)) { + x_191 = lean_alloc_ctor(0, 2, 0); } else { - x_464 = x_462; + x_191 = x_188; } -lean_ctor_set(x_464, 0, x_463); -lean_ctor_set(x_464, 1, x_461); -return x_464; +lean_ctor_set(x_191, 0, x_190); +lean_ctor_set(x_191, 1, x_187); +return x_191; } } } -default: +} +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__1() { +_start: { -lean_object* x_465; lean_object* x_466; -lean_dec(x_3); -lean_dec(x_2); -x_465 = lean_box(0); -x_466 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_466, 0, x_465); -lean_ctor_set(x_466, 1, x_6); -return x_466; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("MutualDef", 9, 9); +return x_1; } } +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("body", 4, 4); +return x_1; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__3() { _start: { -lean_object* x_6; lean_object* x_7; -x_6 = lean_box(0); -x_7 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_7, 0, x_6); -lean_ctor_set(x_7, 1, x_5); -return x_7; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__1; +x_2 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__2; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___closed__1() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__4() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__5___boxed), 5, 0); +x_1 = l_Lean_Linter_linter_unusedVariables_analyzeTactics; return x_1; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__5() { _start: { -uint8_t x_8; -x_8 = lean_usize_dec_lt(x_4, x_3); -if (x_8 == 0) -{ -lean_object* x_9; -lean_dec(x_6); -lean_dec(x_1); -x_9 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_9, 0, x_5); -lean_ctor_set(x_9, 1, x_7); -return x_9; +lean_object* x_1; +x_1 = l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_box(0), lean_box(0)); +return x_1; } -else +} +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__6() { +_start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -lean_dec(x_5); -x_10 = lean_array_uget(x_2, x_4); -lean_inc(x_1); -x_11 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__4___boxed), 6, 1); -lean_closure_set(x_11, 0, x_1); -x_12 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___closed__1; -lean_inc(x_6); -x_13 = l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences___spec__16(x_11, x_12, x_10, x_6, x_7); -if (lean_obj_tag(x_13) == 0) -{ -lean_object* x_14; size_t x_15; size_t x_16; lean_object* x_17; -x_14 = lean_ctor_get(x_13, 1); -lean_inc(x_14); -lean_dec(x_13); -x_15 = 1; -x_16 = lean_usize_add(x_4, x_15); -x_17 = lean_box(0); -x_4 = x_16; -x_5 = x_17; -x_7 = x_14; -goto _start; +lean_object* x_1; lean_object* x_2; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__5; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; } -else +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, lean_object* x_6, lean_object* x_7) { +_start: { -uint8_t x_19; -lean_dec(x_6); +switch (lean_obj_tag(x_3)) { +case 0: +{ +lean_dec(x_2); lean_dec(x_1); -x_19 = !lean_is_exclusive(x_13); -if (x_19 == 0) +if (x_5 == 0) { -return x_13; +lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_8 = lean_ctor_get(x_3, 0); +lean_inc(x_8); +lean_dec(x_3); +x_9 = lean_box(0); +x_10 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__1(x_8, x_9, x_5, x_6, x_7); +lean_dec(x_6); +return x_10; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_13, 0); -x_21 = lean_ctor_get(x_13, 1); -lean_inc(x_21); -lean_inc(x_20); -lean_dec(x_13); -x_22 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_22, 0, x_20); -lean_ctor_set(x_22, 1, x_21); -return x_22; -} -} +uint8_t x_11; lean_object* x_12; lean_object* x_13; +lean_dec(x_6); +lean_dec(x_3); +x_11 = 1; +x_12 = lean_box(x_11); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_7); +return x_13; } } +case 1: +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_14 = lean_ctor_get(x_3, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +lean_dec(x_15); +x_17 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__3; +x_18 = lean_name_eq(x_16, x_17); +lean_dec(x_16); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; +x_19 = lean_box(0); +x_20 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__8(x_5, x_14, x_3, x_2, x_1, x_19, x_5, x_6, x_7); +lean_dec(x_1); +lean_dec(x_3); +return x_20; } -LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_collectReferences(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: +else { -size_t x_5; size_t x_6; lean_object* x_7; lean_object* x_8; -x_5 = lean_array_size(x_1); -x_6 = 0; -x_7 = lean_box(0); -x_8 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21(x_2, x_1, x_5, x_6, x_7, x_3, x_4); -if (lean_obj_tag(x_8) == 0) +lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; +x_21 = lean_ctor_get(x_2, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_21, 3); +lean_inc(x_22); +x_23 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__4; +x_24 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_22, x_23); +lean_dec(x_22); +if (x_24 == 0) { -uint8_t x_9; -x_9 = !lean_is_exclusive(x_8); -if (x_9 == 0) +uint8_t x_25; +x_25 = !lean_is_exclusive(x_3); +if (x_25 == 0) { -lean_object* x_10; -x_10 = lean_ctor_get(x_8, 0); -lean_dec(x_10); -lean_ctor_set(x_8, 0, x_7); -return x_8; +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; +x_26 = lean_ctor_get(x_3, 0); +lean_dec(x_26); +x_27 = lean_ctor_get(x_21, 2); +lean_inc(x_27); +lean_dec(x_21); +x_28 = lean_ctor_get(x_14, 3); +lean_inc(x_28); +lean_dec(x_14); +x_29 = l_Lean_instantiateMVarsCore(x_27, x_28); +x_30 = lean_ctor_get(x_29, 0); +lean_inc(x_30); +lean_dec(x_29); +x_31 = lean_st_ref_take(x_6, x_7); +x_32 = lean_ctor_get(x_31, 0); +lean_inc(x_32); +x_33 = lean_ctor_get(x_31, 1); +lean_inc(x_33); +lean_dec(x_31); +x_34 = !lean_is_exclusive(x_32); +if (x_34 == 0) +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; lean_object* x_43; +x_35 = lean_ctor_get(x_32, 4); +x_36 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__6; +x_37 = lean_box(0); +x_38 = l_Lean_PersistentHashMap_insert___at_Lean_MVarId_assign___spec__1(x_36, x_37, x_30); +x_39 = lean_array_push(x_35, x_38); +lean_ctor_set(x_32, 4, x_39); +x_40 = lean_st_ref_set(x_6, x_32, x_33); +x_41 = lean_ctor_get(x_40, 1); +lean_inc(x_41); +lean_dec(x_40); +x_42 = l_Lean_PersistentArray_anyM___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__11(x_4); +x_43 = l_Lean_PersistentArray_toArray___rarg(x_4); +lean_ctor_set(x_3, 0, x_2); +if (x_5 == 0) +{ +lean_object* x_44; +x_44 = l_Lean_Linter_UnusedVariables_collectReferences_go(x_1, x_43, x_3, x_42, x_6, x_41); +lean_dec(x_43); +if (lean_obj_tag(x_44) == 0) +{ +uint8_t x_45; +x_45 = !lean_is_exclusive(x_44); +if (x_45 == 0) +{ +lean_object* x_46; uint8_t x_47; lean_object* x_48; +x_46 = lean_ctor_get(x_44, 0); +lean_dec(x_46); +x_47 = 0; +x_48 = lean_box(x_47); +lean_ctor_set(x_44, 0, x_48); +return x_44; } else { -lean_object* x_11; lean_object* x_12; -x_11 = lean_ctor_get(x_8, 1); -lean_inc(x_11); -lean_dec(x_8); -x_12 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_12, 0, x_7); -lean_ctor_set(x_12, 1, x_11); -return x_12; +lean_object* x_49; uint8_t x_50; lean_object* x_51; lean_object* x_52; +x_49 = lean_ctor_get(x_44, 1); +lean_inc(x_49); +lean_dec(x_44); +x_50 = 0; +x_51 = lean_box(x_50); +x_52 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_52, 0, x_51); +lean_ctor_set(x_52, 1, x_49); +return x_52; } } else { -uint8_t x_13; -x_13 = !lean_is_exclusive(x_8); -if (x_13 == 0) +uint8_t x_53; +x_53 = !lean_is_exclusive(x_44); +if (x_53 == 0) { -return x_8; +return x_44; } else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_14 = lean_ctor_get(x_8, 0); -x_15 = lean_ctor_get(x_8, 1); -lean_inc(x_15); -lean_inc(x_14); -lean_dec(x_8); -x_16 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_16, 0, x_14); -lean_ctor_set(x_16, 1, x_15); -return x_16; +lean_object* x_54; lean_object* x_55; lean_object* x_56; +x_54 = lean_ctor_get(x_44, 0); +x_55 = lean_ctor_get(x_44, 1); +lean_inc(x_55); +lean_inc(x_54); +lean_dec(x_44); +x_56 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_56, 0, x_54); +lean_ctor_set(x_56, 1, x_55); +return x_56; } } } +else +{ +uint8_t x_57; lean_object* x_58; +x_57 = 1; +x_58 = l_Lean_Linter_UnusedVariables_collectReferences_go(x_1, x_43, x_3, x_57, x_6, x_41); +lean_dec(x_43); +if (lean_obj_tag(x_58) == 0) +{ +uint8_t x_59; +x_59 = !lean_is_exclusive(x_58); +if (x_59 == 0) +{ +lean_object* x_60; uint8_t x_61; lean_object* x_62; +x_60 = lean_ctor_get(x_58, 0); +lean_dec(x_60); +x_61 = 0; +x_62 = lean_box(x_61); +lean_ctor_set(x_58, 0, x_62); +return x_58; } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_collectReferences___spec__1___boxed(lean_object* x_1, lean_object* x_2) { -_start: +else { -lean_object* x_3; -x_3 = l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_collectReferences___spec__1(x_1, x_2); -lean_dec(x_2); -lean_dec(x_1); -return x_3; +lean_object* x_63; uint8_t x_64; lean_object* x_65; lean_object* x_66; +x_63 = lean_ctor_get(x_58, 1); +lean_inc(x_63); +lean_dec(x_58); +x_64 = 0; +x_65 = lean_box(x_64); +x_66 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_66, 0, x_65); +lean_ctor_set(x_66, 1, x_63); +return x_66; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__2___boxed(lean_object* x_1, lean_object* x_2) { -_start: +else { -uint8_t x_3; lean_object* x_4; -x_3 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__2(x_1, x_2); -lean_dec(x_2); -lean_dec(x_1); -x_4 = lean_box(x_3); -return x_4; -} +uint8_t x_67; +x_67 = !lean_is_exclusive(x_58); +if (x_67 == 0) +{ +return x_58; } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__7___boxed(lean_object* x_1, lean_object* x_2) { -_start: +else { -uint8_t x_3; lean_object* x_4; -x_3 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__7(x_1, x_2); -lean_dec(x_2); -lean_dec(x_1); -x_4 = lean_box(x_3); -return x_4; +lean_object* x_68; lean_object* x_69; lean_object* x_70; +x_68 = lean_ctor_get(x_58, 0); +x_69 = lean_ctor_get(x_58, 1); +lean_inc(x_69); +lean_inc(x_68); +lean_dec(x_58); +x_70 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_70, 0, x_68); +lean_ctor_set(x_70, 1, x_69); +return x_70; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__11___boxed(lean_object* x_1, lean_object* x_2) { -_start: -{ -uint8_t x_3; lean_object* x_4; -x_3 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__11(x_1, x_2); -lean_dec(x_2); -lean_dec(x_1); -x_4 = lean_box(x_3); -return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences___spec__16___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: +else { -lean_object* x_8; -x_8 = l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences___spec__16___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -lean_dec(x_5); -return x_8; +lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; uint8_t x_83; lean_object* x_84; +x_71 = lean_ctor_get(x_32, 0); +x_72 = lean_ctor_get(x_32, 1); +x_73 = lean_ctor_get(x_32, 2); +x_74 = lean_ctor_get(x_32, 3); +x_75 = lean_ctor_get(x_32, 4); +lean_inc(x_75); +lean_inc(x_74); +lean_inc(x_73); +lean_inc(x_72); +lean_inc(x_71); +lean_dec(x_32); +x_76 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__6; +x_77 = lean_box(0); +x_78 = l_Lean_PersistentHashMap_insert___at_Lean_MVarId_assign___spec__1(x_76, x_77, x_30); +x_79 = lean_array_push(x_75, x_78); +x_80 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_80, 0, x_71); +lean_ctor_set(x_80, 1, x_72); +lean_ctor_set(x_80, 2, x_73); +lean_ctor_set(x_80, 3, x_74); +lean_ctor_set(x_80, 4, x_79); +x_81 = lean_st_ref_set(x_6, x_80, x_33); +x_82 = lean_ctor_get(x_81, 1); +lean_inc(x_82); +lean_dec(x_81); +x_83 = l_Lean_PersistentArray_anyM___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__11(x_4); +x_84 = l_Lean_PersistentArray_toArray___rarg(x_4); +lean_ctor_set(x_3, 0, x_2); +if (x_5 == 0) +{ +lean_object* x_85; +x_85 = l_Lean_Linter_UnusedVariables_collectReferences_go(x_1, x_84, x_3, x_83, x_6, x_82); +lean_dec(x_84); +if (lean_obj_tag(x_85) == 0) +{ +lean_object* x_86; lean_object* x_87; uint8_t x_88; lean_object* x_89; lean_object* x_90; +x_86 = lean_ctor_get(x_85, 1); +lean_inc(x_86); +if (lean_is_exclusive(x_85)) { + lean_ctor_release(x_85, 0); + lean_ctor_release(x_85, 1); + x_87 = x_85; +} else { + lean_dec_ref(x_85); + x_87 = lean_box(0); +} +x_88 = 0; +x_89 = lean_box(x_88); +if (lean_is_scalar(x_87)) { + x_90 = lean_alloc_ctor(0, 2, 0); +} else { + x_90 = x_87; } +lean_ctor_set(x_90, 0, x_89); +lean_ctor_set(x_90, 1, x_86); +return x_90; } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: +else { -lean_object* x_9; -x_9 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_2); -return x_9; +lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; +x_91 = lean_ctor_get(x_85, 0); +lean_inc(x_91); +x_92 = lean_ctor_get(x_85, 1); +lean_inc(x_92); +if (lean_is_exclusive(x_85)) { + lean_ctor_release(x_85, 0); + lean_ctor_release(x_85, 1); + x_93 = x_85; +} else { + lean_dec_ref(x_85); + x_93 = lean_box(0); } +if (lean_is_scalar(x_93)) { + x_94 = lean_alloc_ctor(1, 2, 0); +} else { + x_94 = x_93; } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; -x_9 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_3); -return x_9; +lean_ctor_set(x_94, 0, x_91); +lean_ctor_set(x_94, 1, x_92); +return x_94; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: +else { -lean_object* x_9; -x_9 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_4); -return x_9; +uint8_t x_95; lean_object* x_96; +x_95 = 1; +x_96 = l_Lean_Linter_UnusedVariables_collectReferences_go(x_1, x_84, x_3, x_95, x_6, x_82); +lean_dec(x_84); +if (lean_obj_tag(x_96) == 0) +{ +lean_object* x_97; lean_object* x_98; uint8_t x_99; lean_object* x_100; lean_object* x_101; +x_97 = lean_ctor_get(x_96, 1); +lean_inc(x_97); +if (lean_is_exclusive(x_96)) { + lean_ctor_release(x_96, 0); + lean_ctor_release(x_96, 1); + x_98 = x_96; +} else { + lean_dec_ref(x_96); + x_98 = lean_box(0); } +x_99 = 0; +x_100 = lean_box(x_99); +if (lean_is_scalar(x_98)) { + x_101 = lean_alloc_ctor(0, 2, 0); +} else { + x_101 = x_98; } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: +lean_ctor_set(x_101, 0, x_100); +lean_ctor_set(x_101, 1, x_97); +return x_101; +} +else { -lean_object* x_7; -x_7 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_1); -return x_7; +lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; +x_102 = lean_ctor_get(x_96, 0); +lean_inc(x_102); +x_103 = lean_ctor_get(x_96, 1); +lean_inc(x_103); +if (lean_is_exclusive(x_96)) { + lean_ctor_release(x_96, 0); + lean_ctor_release(x_96, 1); + x_104 = x_96; +} else { + lean_dec_ref(x_96); + x_104 = lean_box(0); } +if (lean_is_scalar(x_104)) { + x_105 = lean_alloc_ctor(1, 2, 0); +} else { + x_105 = x_104; } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: +lean_ctor_set(x_105, 0, x_102); +lean_ctor_set(x_105, 1, x_103); +return x_105; +} +} +} +} +else { -lean_object* x_6; -x_6 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__5(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_4); +lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; uint8_t x_126; lean_object* x_127; lean_object* x_128; +lean_dec(x_3); +x_106 = lean_ctor_get(x_21, 2); +lean_inc(x_106); +lean_dec(x_21); +x_107 = lean_ctor_get(x_14, 3); +lean_inc(x_107); +lean_dec(x_14); +x_108 = l_Lean_instantiateMVarsCore(x_106, x_107); +x_109 = lean_ctor_get(x_108, 0); +lean_inc(x_109); +lean_dec(x_108); +x_110 = lean_st_ref_take(x_6, x_7); +x_111 = lean_ctor_get(x_110, 0); +lean_inc(x_111); +x_112 = lean_ctor_get(x_110, 1); +lean_inc(x_112); +lean_dec(x_110); +x_113 = lean_ctor_get(x_111, 0); +lean_inc(x_113); +x_114 = lean_ctor_get(x_111, 1); +lean_inc(x_114); +x_115 = lean_ctor_get(x_111, 2); +lean_inc(x_115); +x_116 = lean_ctor_get(x_111, 3); +lean_inc(x_116); +x_117 = lean_ctor_get(x_111, 4); +lean_inc(x_117); +if (lean_is_exclusive(x_111)) { + lean_ctor_release(x_111, 0); + lean_ctor_release(x_111, 1); + lean_ctor_release(x_111, 2); + lean_ctor_release(x_111, 3); + lean_ctor_release(x_111, 4); + x_118 = x_111; +} else { + lean_dec_ref(x_111); + x_118 = lean_box(0); +} +x_119 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__6; +x_120 = lean_box(0); +x_121 = l_Lean_PersistentHashMap_insert___at_Lean_MVarId_assign___spec__1(x_119, x_120, x_109); +x_122 = lean_array_push(x_117, x_121); +if (lean_is_scalar(x_118)) { + x_123 = lean_alloc_ctor(0, 5, 0); +} else { + x_123 = x_118; +} +lean_ctor_set(x_123, 0, x_113); +lean_ctor_set(x_123, 1, x_114); +lean_ctor_set(x_123, 2, x_115); +lean_ctor_set(x_123, 3, x_116); +lean_ctor_set(x_123, 4, x_122); +x_124 = lean_st_ref_set(x_6, x_123, x_112); +x_125 = lean_ctor_get(x_124, 1); +lean_inc(x_125); +lean_dec(x_124); +x_126 = l_Lean_PersistentArray_anyM___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__11(x_4); +x_127 = l_Lean_PersistentArray_toArray___rarg(x_4); +x_128 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_128, 0, x_2); +if (x_5 == 0) +{ +lean_object* x_129; +x_129 = l_Lean_Linter_UnusedVariables_collectReferences_go(x_1, x_127, x_128, x_126, x_6, x_125); +lean_dec(x_127); +if (lean_obj_tag(x_129) == 0) +{ +lean_object* x_130; lean_object* x_131; uint8_t x_132; lean_object* x_133; lean_object* x_134; +x_130 = lean_ctor_get(x_129, 1); +lean_inc(x_130); +if (lean_is_exclusive(x_129)) { + lean_ctor_release(x_129, 0); + lean_ctor_release(x_129, 1); + x_131 = x_129; +} else { + lean_dec_ref(x_129); + x_131 = lean_box(0); +} +x_132 = 0; +x_133 = lean_box(x_132); +if (lean_is_scalar(x_131)) { + x_134 = lean_alloc_ctor(0, 2, 0); +} else { + x_134 = x_131; +} +lean_ctor_set(x_134, 0, x_133); +lean_ctor_set(x_134, 1, x_130); +return x_134; +} +else +{ +lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; +x_135 = lean_ctor_get(x_129, 0); +lean_inc(x_135); +x_136 = lean_ctor_get(x_129, 1); +lean_inc(x_136); +if (lean_is_exclusive(x_129)) { + lean_ctor_release(x_129, 0); + lean_ctor_release(x_129, 1); + x_137 = x_129; +} else { + lean_dec_ref(x_129); + x_137 = lean_box(0); +} +if (lean_is_scalar(x_137)) { + x_138 = lean_alloc_ctor(1, 2, 0); +} else { + x_138 = x_137; +} +lean_ctor_set(x_138, 0, x_135); +lean_ctor_set(x_138, 1, x_136); +return x_138; +} +} +else +{ +uint8_t x_139; lean_object* x_140; +x_139 = 1; +x_140 = l_Lean_Linter_UnusedVariables_collectReferences_go(x_1, x_127, x_128, x_139, x_6, x_125); +lean_dec(x_127); +if (lean_obj_tag(x_140) == 0) +{ +lean_object* x_141; lean_object* x_142; uint8_t x_143; lean_object* x_144; lean_object* x_145; +x_141 = lean_ctor_get(x_140, 1); +lean_inc(x_141); +if (lean_is_exclusive(x_140)) { + lean_ctor_release(x_140, 0); + lean_ctor_release(x_140, 1); + x_142 = x_140; +} else { + lean_dec_ref(x_140); + x_142 = lean_box(0); +} +x_143 = 0; +x_144 = lean_box(x_143); +if (lean_is_scalar(x_142)) { + x_145 = lean_alloc_ctor(0, 2, 0); +} else { + x_145 = x_142; +} +lean_ctor_set(x_145, 0, x_144); +lean_ctor_set(x_145, 1, x_141); +return x_145; +} +else +{ +lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; +x_146 = lean_ctor_get(x_140, 0); +lean_inc(x_146); +x_147 = lean_ctor_get(x_140, 1); +lean_inc(x_147); +if (lean_is_exclusive(x_140)) { + lean_ctor_release(x_140, 0); + lean_ctor_release(x_140, 1); + x_148 = x_140; +} else { + lean_dec_ref(x_140); + x_148 = lean_box(0); +} +if (lean_is_scalar(x_148)) { + x_149 = lean_alloc_ctor(1, 2, 0); +} else { + x_149 = x_148; +} +lean_ctor_set(x_149, 0, x_146); +lean_ctor_set(x_149, 1, x_147); +return x_149; +} +} +} +} +else +{ +lean_object* x_150; lean_object* x_151; +lean_dec(x_21); +x_150 = lean_box(0); +x_151 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__8(x_5, x_14, x_3, x_2, x_1, x_150, x_5, x_6, x_7); +lean_dec(x_1); lean_dec(x_3); +return x_151; +} +} +} +case 9: +{ lean_dec(x_2); lean_dec(x_1); -return x_6; +if (x_5 == 0) +{ +lean_object* x_152; lean_object* x_153; lean_object* x_154; +x_152 = lean_ctor_get(x_3, 0); +lean_inc(x_152); +lean_dec(x_3); +x_153 = lean_box(0); +x_154 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__9(x_152, x_153, x_5, x_6, x_7); +lean_dec(x_6); +return x_154; } +else +{ +uint8_t x_155; lean_object* x_156; lean_object* x_157; +lean_dec(x_6); +lean_dec(x_3); +x_155 = 1; +x_156 = lean_box(x_155); +x_157 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_157, 0, x_156); +lean_ctor_set(x_157, 1, x_7); +return x_157; } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: +} +default: { -size_t x_8; size_t x_9; lean_object* x_10; -x_8 = lean_unbox_usize(x_3); +uint8_t x_158; lean_object* x_159; lean_object* x_160; +lean_dec(x_6); lean_dec(x_3); -x_9 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_10 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21(x_1, x_2, x_8, x_9, x_5, x_6, x_7); lean_dec(x_2); -return x_10; +lean_dec(x_1); +x_158 = 1; +x_159 = lean_box(x_158); +x_160 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_160, 0, x_159); +lean_ctor_set(x_160, 1, x_7); +return x_160; } } -LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_collectReferences___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__11(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6) { _start: { -lean_object* x_5; -x_5 = l_Lean_Linter_UnusedVariables_collectReferences(x_1, x_2, x_3, x_4); -lean_dec(x_1); -return x_5; +lean_object* x_7; lean_object* x_8; +x_7 = lean_box(0); +x_8 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_8, 0, x_7); +lean_ctor_set(x_8, 1, x_6); +return x_8; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___closed__1() { _start: { -if (lean_obj_tag(x_4) == 0) +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__11___boxed), 6, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6, uint8_t x_7, lean_object* x_8, lean_object* x_9) { +_start: { +uint8_t x_10; +x_10 = lean_usize_dec_lt(x_5, x_4); +if (x_10 == 0) +{ +lean_object* x_11; +lean_dec(x_8); +lean_dec(x_2); lean_dec(x_1); -return x_3; +x_11 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_11, 0, x_6); +lean_ctor_set(x_11, 1, x_9); +return x_11; } else { -uint8_t x_5; -x_5 = !lean_is_exclusive(x_4); -if (x_5 == 0) -{ -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; -x_6 = lean_ctor_get(x_4, 0); -x_7 = lean_ctor_get(x_4, 1); -x_8 = lean_ctor_get(x_4, 2); -x_9 = lean_ctor_get(x_2, 3); -x_10 = l_Lean_Linter_UnusedVariables_followAliases(x_9, x_7); -x_11 = !lean_is_exclusive(x_3); -if (x_11 == 0) -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; uint64_t x_15; uint64_t x_16; uint64_t x_17; uint64_t x_18; uint64_t x_19; uint64_t x_20; uint64_t x_21; size_t x_22; size_t x_23; size_t x_24; size_t x_25; size_t x_26; lean_object* x_27; uint8_t x_28; -x_12 = lean_ctor_get(x_3, 0); -x_13 = lean_ctor_get(x_3, 1); -x_14 = lean_array_get_size(x_13); -x_15 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_6); -x_16 = 32; -x_17 = lean_uint64_shift_right(x_15, x_16); -x_18 = lean_uint64_xor(x_15, x_17); -x_19 = 16; -x_20 = lean_uint64_shift_right(x_18, x_19); -x_21 = lean_uint64_xor(x_18, x_20); -x_22 = lean_uint64_to_usize(x_21); -x_23 = lean_usize_of_nat(x_14); -lean_dec(x_14); -x_24 = 1; -x_25 = lean_usize_sub(x_23, x_24); -x_26 = lean_usize_land(x_22, x_25); -x_27 = lean_array_uget(x_13, x_26); -x_28 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__11(x_6, x_27); -if (x_28 == 0) -{ -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; -x_29 = lean_unsigned_to_nat(1u); -x_30 = lean_nat_add(x_12, x_29); -lean_dec(x_12); -lean_ctor_set(x_4, 2, x_27); -lean_ctor_set(x_4, 1, x_10); -x_31 = lean_array_uset(x_13, x_26, x_4); -x_32 = lean_unsigned_to_nat(4u); -x_33 = lean_nat_mul(x_30, x_32); -x_34 = lean_unsigned_to_nat(3u); -x_35 = lean_nat_div(x_33, x_34); -lean_dec(x_33); -x_36 = lean_array_get_size(x_31); -x_37 = lean_nat_dec_le(x_35, x_36); -lean_dec(x_36); -lean_dec(x_35); -if (x_37 == 0) +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_dec(x_6); +x_12 = lean_array_uget(x_3, x_5); +lean_inc(x_1); +x_13 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___boxed), 7, 1); +lean_closure_set(x_13, 0, x_1); +x_14 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___closed__1; +lean_inc(x_8); +lean_inc(x_2); +x_15 = l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__20(x_13, x_14, x_2, x_12, x_7, x_8, x_9); +if (lean_obj_tag(x_15) == 0) { -lean_object* x_38; -x_38 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__12(x_31); -lean_ctor_set(x_3, 1, x_38); -lean_ctor_set(x_3, 0, x_30); -x_4 = x_8; +lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; +x_16 = lean_ctor_get(x_15, 1); +lean_inc(x_16); +lean_dec(x_15); +x_17 = 1; +x_18 = lean_usize_add(x_5, x_17); +x_19 = lean_box(0); +x_5 = x_18; +x_6 = x_19; +x_9 = x_16; goto _start; } else { -lean_ctor_set(x_3, 1, x_31); -lean_ctor_set(x_3, 0, x_30); -x_4 = x_8; -goto _start; -} +uint8_t x_21; +lean_dec(x_8); +lean_dec(x_2); +lean_dec(x_1); +x_21 = !lean_is_exclusive(x_15); +if (x_21 == 0) +{ +return x_15; } else { -lean_object* x_41; lean_object* x_42; lean_object* x_43; -lean_free_object(x_4); -lean_inc(x_1); -x_41 = lean_array_uset(x_13, x_26, x_1); -x_42 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__15(x_6, x_10, x_27); -x_43 = lean_array_uset(x_41, x_26, x_42); -lean_ctor_set(x_3, 1, x_43); -x_4 = x_8; -goto _start; +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_15, 0); +x_23 = lean_ctor_get(x_15, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_15); +x_24 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); +return x_24; } } -else +} +} +} +LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_collectReferences_go(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6) { +_start: { -lean_object* x_45; lean_object* x_46; lean_object* x_47; uint64_t x_48; uint64_t x_49; uint64_t x_50; uint64_t x_51; uint64_t x_52; uint64_t x_53; uint64_t x_54; size_t x_55; size_t x_56; size_t x_57; size_t x_58; size_t x_59; lean_object* x_60; uint8_t x_61; -x_45 = lean_ctor_get(x_3, 0); -x_46 = lean_ctor_get(x_3, 1); -lean_inc(x_46); -lean_inc(x_45); -lean_dec(x_3); -x_47 = lean_array_get_size(x_46); -x_48 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_6); -x_49 = 32; -x_50 = lean_uint64_shift_right(x_48, x_49); -x_51 = lean_uint64_xor(x_48, x_50); -x_52 = 16; -x_53 = lean_uint64_shift_right(x_51, x_52); -x_54 = lean_uint64_xor(x_51, x_53); -x_55 = lean_uint64_to_usize(x_54); -x_56 = lean_usize_of_nat(x_47); -lean_dec(x_47); -x_57 = 1; -x_58 = lean_usize_sub(x_56, x_57); -x_59 = lean_usize_land(x_55, x_58); -x_60 = lean_array_uget(x_46, x_59); -x_61 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__11(x_6, x_60); -if (x_61 == 0) +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = lean_array_size(x_2); +x_8 = 0; +x_9 = lean_box(0); +x_10 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24(x_1, x_3, x_2, x_7, x_8, x_9, x_4, x_5, x_6); +if (lean_obj_tag(x_10) == 0) { -lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; uint8_t x_70; -x_62 = lean_unsigned_to_nat(1u); -x_63 = lean_nat_add(x_45, x_62); -lean_dec(x_45); -lean_ctor_set(x_4, 2, x_60); -lean_ctor_set(x_4, 1, x_10); -x_64 = lean_array_uset(x_46, x_59, x_4); -x_65 = lean_unsigned_to_nat(4u); -x_66 = lean_nat_mul(x_63, x_65); -x_67 = lean_unsigned_to_nat(3u); -x_68 = lean_nat_div(x_66, x_67); -lean_dec(x_66); -x_69 = lean_array_get_size(x_64); -x_70 = lean_nat_dec_le(x_68, x_69); -lean_dec(x_69); -lean_dec(x_68); -if (x_70 == 0) +uint8_t x_11; +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) { -lean_object* x_71; lean_object* x_72; -x_71 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__12(x_64); -x_72 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_72, 0, x_63); -lean_ctor_set(x_72, 1, x_71); -x_3 = x_72; -x_4 = x_8; -goto _start; +lean_object* x_12; +x_12 = lean_ctor_get(x_10, 0); +lean_dec(x_12); +lean_ctor_set(x_10, 0, x_9); +return x_10; } else { -lean_object* x_74; -x_74 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_74, 0, x_63); -lean_ctor_set(x_74, 1, x_64); -x_3 = x_74; -x_4 = x_8; -goto _start; +lean_object* x_13; lean_object* x_14; +x_13 = lean_ctor_get(x_10, 1); +lean_inc(x_13); +lean_dec(x_10); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_9); +lean_ctor_set(x_14, 1, x_13); +return x_14; } } else { -lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; -lean_free_object(x_4); -lean_inc(x_1); -x_76 = lean_array_uset(x_46, x_59, x_1); -x_77 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__15(x_6, x_10, x_60); -x_78 = lean_array_uset(x_76, x_59, x_77); -x_79 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_79, 0, x_45); -lean_ctor_set(x_79, 1, x_78); -x_3 = x_79; -x_4 = x_8; -goto _start; -} -} +uint8_t x_15; +x_15 = !lean_is_exclusive(x_10); +if (x_15 == 0) +{ +return x_10; } else { -lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; uint64_t x_90; uint64_t x_91; uint64_t x_92; uint64_t x_93; uint64_t x_94; uint64_t x_95; uint64_t x_96; size_t x_97; size_t x_98; size_t x_99; size_t x_100; size_t x_101; lean_object* x_102; uint8_t x_103; -x_81 = lean_ctor_get(x_4, 0); -x_82 = lean_ctor_get(x_4, 1); -x_83 = lean_ctor_get(x_4, 2); -lean_inc(x_83); -lean_inc(x_82); -lean_inc(x_81); -lean_dec(x_4); -x_84 = lean_ctor_get(x_2, 3); -x_85 = l_Lean_Linter_UnusedVariables_followAliases(x_84, x_82); -x_86 = lean_ctor_get(x_3, 0); -lean_inc(x_86); -x_87 = lean_ctor_get(x_3, 1); -lean_inc(x_87); -if (lean_is_exclusive(x_3)) { - lean_ctor_release(x_3, 0); - lean_ctor_release(x_3, 1); - x_88 = x_3; -} else { - lean_dec_ref(x_3); - x_88 = lean_box(0); +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_10, 0); +x_17 = lean_ctor_get(x_10, 1); +lean_inc(x_17); +lean_inc(x_16); +lean_dec(x_10); +x_18 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_18, 0, x_16); +lean_ctor_set(x_18, 1, x_17); +return x_18; } -x_89 = lean_array_get_size(x_87); -x_90 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_81); -x_91 = 32; -x_92 = lean_uint64_shift_right(x_90, x_91); -x_93 = lean_uint64_xor(x_90, x_92); -x_94 = 16; -x_95 = lean_uint64_shift_right(x_93, x_94); -x_96 = lean_uint64_xor(x_93, x_95); -x_97 = lean_uint64_to_usize(x_96); -x_98 = lean_usize_of_nat(x_89); -lean_dec(x_89); -x_99 = 1; -x_100 = lean_usize_sub(x_98, x_99); -x_101 = lean_usize_land(x_97, x_100); -x_102 = lean_array_uget(x_87, x_101); -x_103 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__11(x_81, x_102); -if (x_103 == 0) +} +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__1___boxed(lean_object* x_1, lean_object* x_2) { +_start: { -lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; uint8_t x_113; -x_104 = lean_unsigned_to_nat(1u); -x_105 = lean_nat_add(x_86, x_104); -lean_dec(x_86); -x_106 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_106, 0, x_81); -lean_ctor_set(x_106, 1, x_85); -lean_ctor_set(x_106, 2, x_102); -x_107 = lean_array_uset(x_87, x_101, x_106); -x_108 = lean_unsigned_to_nat(4u); -x_109 = lean_nat_mul(x_105, x_108); -x_110 = lean_unsigned_to_nat(3u); -x_111 = lean_nat_div(x_109, x_110); -lean_dec(x_109); -x_112 = lean_array_get_size(x_107); -x_113 = lean_nat_dec_le(x_111, x_112); -lean_dec(x_112); -lean_dec(x_111); -if (x_113 == 0) +lean_object* x_3; +x_3 = l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__1(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__2___boxed(lean_object* x_1, lean_object* x_2) { +_start: { -lean_object* x_114; lean_object* x_115; -x_114 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__12(x_107); -if (lean_is_scalar(x_88)) { - x_115 = lean_alloc_ctor(0, 2, 0); -} else { - x_115 = x_88; +uint8_t x_3; lean_object* x_4; +x_3 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__2(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +x_4 = lean_box(x_3); +return x_4; } -lean_ctor_set(x_115, 0, x_105); -lean_ctor_set(x_115, 1, x_114); -x_3 = x_115; -x_4 = x_83; -goto _start; } -else +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__7___boxed(lean_object* x_1, lean_object* x_2) { +_start: { -lean_object* x_117; -if (lean_is_scalar(x_88)) { - x_117 = lean_alloc_ctor(0, 2, 0); -} else { - x_117 = x_88; +uint8_t x_3; lean_object* x_4; +x_3 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__7(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +x_4 = lean_box(x_3); +return x_4; } -lean_ctor_set(x_117, 0, x_105); -lean_ctor_set(x_117, 1, x_107); -x_3 = x_117; -x_4 = x_83; -goto _start; +} +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; size_t x_5; uint8_t x_6; lean_object* x_7; +x_4 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_5 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_6 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__13(x_1, x_4, x_5); +lean_dec(x_1); +x_7 = lean_box(x_6); +return x_7; } } -else +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14___lambda__1___boxed(lean_object* x_1) { +_start: { -lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; -lean_inc(x_1); -x_119 = lean_array_uset(x_87, x_101, x_1); -x_120 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__15(x_81, x_85, x_102); -x_121 = lean_array_uset(x_119, x_101, x_120); -if (lean_is_scalar(x_88)) { - x_122 = lean_alloc_ctor(0, 2, 0); -} else { - x_122 = x_88; +uint8_t x_2; lean_object* x_3; +x_2 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14___lambda__1(x_1); +lean_dec(x_1); +x_3 = lean_box(x_2); +return x_3; } -lean_ctor_set(x_122, 0, x_86); -lean_ctor_set(x_122, 1, x_121); -x_3 = x_122; -x_4 = x_83; -goto _start; } +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; size_t x_5; uint8_t x_6; lean_object* x_7; +x_4 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_5 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_6 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14(x_1, x_4, x_5); +lean_dec(x_1); +x_7 = lean_box(x_6); +return x_7; } } +LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__12___boxed(lean_object* x_1) { +_start: +{ +uint8_t x_2; lean_object* x_3; +x_2 = l_Lean_PersistentArray_anyMAux___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__12(x_1); +lean_dec(x_1); +x_3 = lean_box(x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__2(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__11___boxed(lean_object* x_1) { _start: { -if (lean_obj_tag(x_2) == 0) +uint8_t x_2; lean_object* x_3; +x_2 = l_Lean_PersistentArray_anyM___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__11(x_1); +lean_dec(x_1); +x_3 = lean_box(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__15___boxed(lean_object* x_1, lean_object* x_2) { +_start: { -return x_1; +uint8_t x_3; lean_object* x_4; +x_3 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__15(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +x_4 = lean_box(x_3); +return x_4; } -else +} +LEAN_EXPORT lean_object* l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: { -uint8_t x_3; -x_3 = !lean_is_exclusive(x_2); -if (x_3 == 0) +uint8_t x_5; lean_object* x_6; +x_5 = lean_unbox(x_2); +lean_dec(x_2); +x_6 = l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22(x_1, x_5, x_3, x_4); +return x_6; +} +} +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__23___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: { -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; uint64_t x_10; uint64_t x_11; uint64_t x_12; uint64_t x_13; uint64_t x_14; uint64_t x_15; uint64_t x_16; size_t x_17; size_t x_18; size_t x_19; size_t x_20; size_t x_21; lean_object* x_22; uint8_t x_23; -x_4 = lean_ctor_get(x_2, 0); -x_5 = lean_ctor_get(x_2, 1); -x_6 = lean_ctor_get(x_2, 2); -x_7 = lean_ctor_get(x_1, 0); -lean_inc(x_7); -x_8 = lean_ctor_get(x_1, 1); -lean_inc(x_8); -x_9 = lean_array_get_size(x_8); -x_10 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_4); -x_11 = 32; -x_12 = lean_uint64_shift_right(x_10, x_11); -x_13 = lean_uint64_xor(x_10, x_12); -x_14 = 16; -x_15 = lean_uint64_shift_right(x_13, x_14); -x_16 = lean_uint64_xor(x_13, x_15); -x_17 = lean_uint64_to_usize(x_16); -x_18 = lean_usize_of_nat(x_9); -lean_dec(x_9); -x_19 = 1; -x_20 = lean_usize_sub(x_18, x_19); -x_21 = lean_usize_land(x_17, x_20); -x_22 = lean_array_uget(x_8, x_21); -x_23 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_4, x_22); -lean_dec(x_22); -lean_dec(x_4); -if (x_23 == 0) +uint8_t x_9; lean_object* x_10; +x_9 = lean_unbox(x_6); +lean_dec(x_6); +x_10 = l_List_mapM_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__23(x_1, x_2, x_3, x_4, x_5, x_9, x_7, x_8); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: { -lean_dec(x_8); -lean_dec(x_7); -lean_free_object(x_2); +uint8_t x_8; lean_object* x_9; +x_8 = lean_unbox(x_5); lean_dec(x_5); -x_2 = x_6; -goto _start; +x_9 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21(x_1, x_2, x_3, x_4, x_8, x_6, x_7); +return x_9; } -else +} +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__20___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: { -uint8_t x_25; -x_25 = !lean_is_exclusive(x_1); -if (x_25 == 0) +uint8_t x_9; lean_object* x_10; +x_9 = lean_unbox(x_6); +lean_dec(x_6); +x_10 = l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__20___lambda__1(x_1, x_2, x_3, x_4, x_5, x_9, x_7, x_8); +lean_dec(x_5); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__20___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: { -lean_object* x_26; lean_object* x_27; uint64_t x_28; uint64_t x_29; uint64_t x_30; uint64_t x_31; uint64_t x_32; size_t x_33; size_t x_34; lean_object* x_35; uint8_t x_36; -x_26 = lean_ctor_get(x_1, 1); -lean_dec(x_26); -x_27 = lean_ctor_get(x_1, 0); -lean_dec(x_27); -x_28 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_5); -x_29 = lean_uint64_shift_right(x_28, x_11); -x_30 = lean_uint64_xor(x_28, x_29); -x_31 = lean_uint64_shift_right(x_30, x_14); -x_32 = lean_uint64_xor(x_30, x_31); -x_33 = lean_uint64_to_usize(x_32); -x_34 = lean_usize_land(x_33, x_20); -x_35 = lean_array_uget(x_8, x_34); -x_36 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_5, x_35); -if (x_36 == 0) +uint8_t x_8; lean_object* x_9; +x_8 = lean_unbox(x_5); +lean_dec(x_5); +x_9 = l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__20(x_1, x_2, x_3, x_4, x_8, x_6, x_7); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: { -lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; uint8_t x_46; -x_37 = lean_unsigned_to_nat(1u); -x_38 = lean_nat_add(x_7, x_37); +uint8_t x_6; lean_object* x_7; +x_6 = lean_unbox(x_3); +lean_dec(x_3); +x_7 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__1(x_1, x_2, x_6, x_4, x_5); +lean_dec(x_4); +lean_dec(x_2); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; lean_object* x_6; +x_5 = lean_unbox(x_2); +lean_dec(x_2); +x_6 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__2(x_1, x_5, x_3, x_4); +lean_dec(x_3); +lean_dec(x_1); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +uint8_t x_11; lean_object* x_12; +x_11 = lean_unbox(x_8); +lean_dec(x_8); +x_12 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_11, x_9, x_10); lean_dec(x_7); -x_39 = lean_box(0); -lean_ctor_set(x_2, 2, x_35); -lean_ctor_set(x_2, 1, x_39); -lean_ctor_set(x_2, 0, x_5); -x_40 = lean_array_uset(x_8, x_34, x_2); -x_41 = lean_unsigned_to_nat(4u); -x_42 = lean_nat_mul(x_38, x_41); -x_43 = lean_unsigned_to_nat(3u); -x_44 = lean_nat_div(x_42, x_43); -lean_dec(x_42); -x_45 = lean_array_get_size(x_40); -x_46 = lean_nat_dec_le(x_44, x_45); -lean_dec(x_45); -lean_dec(x_44); -if (x_46 == 0) +lean_dec(x_3); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: { -lean_object* x_47; -x_47 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_40); -lean_ctor_set(x_1, 1, x_47); -lean_ctor_set(x_1, 0, x_38); -x_2 = x_6; -goto _start; +uint8_t x_11; lean_object* x_12; +x_11 = lean_unbox(x_8); +lean_dec(x_8); +x_12 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_11, x_9, x_10); +lean_dec(x_7); +lean_dec(x_4); +return x_12; } -else +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: { -lean_ctor_set(x_1, 1, x_40); -lean_ctor_set(x_1, 0, x_38); -x_2 = x_6; -goto _start; +uint8_t x_11; lean_object* x_12; +x_11 = lean_unbox(x_8); +lean_dec(x_8); +x_12 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_11, x_9, x_10); +lean_dec(x_7); +lean_dec(x_5); +return x_12; } } -else +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: { -lean_dec(x_35); -lean_free_object(x_2); +uint8_t x_12; lean_object* x_13; +x_12 = lean_unbox(x_9); +lean_dec(x_9); +x_13 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_12, x_10, x_11); +lean_dec(x_8); +lean_dec(x_7); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +uint8_t x_10; uint8_t x_11; lean_object* x_12; +x_10 = lean_unbox(x_3); +lean_dec(x_3); +x_11 = lean_unbox(x_7); +lean_dec(x_7); +x_12 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__7(x_1, x_2, x_10, x_4, x_5, x_6, x_11, x_8, x_9); +lean_dec(x_6); lean_dec(x_5); -x_2 = x_6; -goto _start; +lean_dec(x_2); +return x_12; } } -else +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: { -uint64_t x_51; uint64_t x_52; uint64_t x_53; uint64_t x_54; uint64_t x_55; size_t x_56; size_t x_57; lean_object* x_58; uint8_t x_59; +uint8_t x_10; uint8_t x_11; lean_object* x_12; +x_10 = lean_unbox(x_1); lean_dec(x_1); -x_51 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_5); -x_52 = lean_uint64_shift_right(x_51, x_11); -x_53 = lean_uint64_xor(x_51, x_52); -x_54 = lean_uint64_shift_right(x_53, x_14); -x_55 = lean_uint64_xor(x_53, x_54); -x_56 = lean_uint64_to_usize(x_55); -x_57 = lean_usize_land(x_56, x_20); -x_58 = lean_array_uget(x_8, x_57); -x_59 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_5, x_58); -if (x_59 == 0) -{ -lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; uint8_t x_69; -x_60 = lean_unsigned_to_nat(1u); -x_61 = lean_nat_add(x_7, x_60); +x_11 = lean_unbox(x_7); lean_dec(x_7); -x_62 = lean_box(0); -lean_ctor_set(x_2, 2, x_58); -lean_ctor_set(x_2, 1, x_62); -lean_ctor_set(x_2, 0, x_5); -x_63 = lean_array_uset(x_8, x_57, x_2); -x_64 = lean_unsigned_to_nat(4u); -x_65 = lean_nat_mul(x_61, x_64); -x_66 = lean_unsigned_to_nat(3u); -x_67 = lean_nat_div(x_65, x_66); -lean_dec(x_65); -x_68 = lean_array_get_size(x_63); -x_69 = lean_nat_dec_le(x_67, x_68); -lean_dec(x_68); -lean_dec(x_67); -if (x_69 == 0) +x_12 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__8(x_10, x_2, x_3, x_4, x_5, x_6, x_11, x_8, x_9); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: { -lean_object* x_70; lean_object* x_71; -x_70 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_63); -x_71 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_71, 0, x_61); -lean_ctor_set(x_71, 1, x_70); -x_1 = x_71; -x_2 = x_6; -goto _start; +uint8_t x_6; lean_object* x_7; +x_6 = lean_unbox(x_3); +lean_dec(x_3); +x_7 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__9(x_1, x_2, x_6, x_4, x_5); +lean_dec(x_4); +lean_dec(x_2); +return x_7; } -else +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: { -lean_object* x_73; -x_73 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_73, 0, x_61); -lean_ctor_set(x_73, 1, x_63); -x_1 = x_73; -x_2 = x_6; -goto _start; +uint8_t x_8; lean_object* x_9; +x_8 = lean_unbox(x_5); +lean_dec(x_5); +x_9 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10(x_1, x_2, x_3, x_4, x_8, x_6, x_7); +lean_dec(x_4); +return x_9; } } -else +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: { -lean_object* x_75; -lean_dec(x_58); -lean_free_object(x_2); +uint8_t x_7; lean_object* x_8; +x_7 = lean_unbox(x_4); +lean_dec(x_4); +x_8 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__11(x_1, x_2, x_3, x_7, x_5, x_6); lean_dec(x_5); -x_75 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_75, 0, x_7); -lean_ctor_set(x_75, 1, x_8); -x_1 = x_75; -x_2 = x_6; -goto _start; +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_8; } } +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +size_t x_10; size_t x_11; uint8_t x_12; lean_object* x_13; +x_10 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_11 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_12 = lean_unbox(x_7); +lean_dec(x_7); +x_13 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24(x_1, x_2, x_3, x_10, x_11, x_6, x_12, x_8, x_9); +lean_dec(x_3); +return x_13; } } -else +LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_collectReferences_go___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: { -lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; uint64_t x_83; uint64_t x_84; uint64_t x_85; uint64_t x_86; uint64_t x_87; uint64_t x_88; uint64_t x_89; size_t x_90; size_t x_91; size_t x_92; size_t x_93; size_t x_94; lean_object* x_95; uint8_t x_96; -x_77 = lean_ctor_get(x_2, 0); +uint8_t x_7; lean_object* x_8; +x_7 = lean_unbox(x_4); +lean_dec(x_4); +x_8 = l_Lean_Linter_UnusedVariables_collectReferences_go(x_1, x_2, x_3, x_7, x_5, x_6); +lean_dec(x_2); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_collectReferences(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; uint8_t x_6; lean_object* x_7; +x_5 = lean_box(0); +x_6 = 0; +x_7 = l_Lean_Linter_UnusedVariables_collectReferences_go(x_2, x_1, x_5, x_6, x_3, x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_collectReferences___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Lean_Linter_UnusedVariables_collectReferences(x_1, x_2, x_3, x_4); +lean_dec(x_1); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +if (lean_obj_tag(x_4) == 0) +{ +lean_dec(x_1); +return x_3; +} +else +{ +uint8_t x_5; +x_5 = !lean_is_exclusive(x_4); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_6 = lean_ctor_get(x_4, 0); +x_7 = lean_ctor_get(x_4, 1); +x_8 = lean_ctor_get(x_4, 2); +x_9 = lean_ctor_get(x_2, 3); +x_10 = l_Lean_Linter_UnusedVariables_followAliases(x_9, x_7); +x_11 = !lean_is_exclusive(x_3); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; uint64_t x_15; uint64_t x_16; uint64_t x_17; uint64_t x_18; uint64_t x_19; uint64_t x_20; uint64_t x_21; size_t x_22; size_t x_23; size_t x_24; size_t x_25; size_t x_26; lean_object* x_27; uint8_t x_28; +x_12 = lean_ctor_get(x_3, 0); +x_13 = lean_ctor_get(x_3, 1); +x_14 = lean_array_get_size(x_13); +x_15 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_6); +x_16 = 32; +x_17 = lean_uint64_shift_right(x_15, x_16); +x_18 = lean_uint64_xor(x_15, x_17); +x_19 = 16; +x_20 = lean_uint64_shift_right(x_18, x_19); +x_21 = lean_uint64_xor(x_18, x_20); +x_22 = lean_uint64_to_usize(x_21); +x_23 = lean_usize_of_nat(x_14); +lean_dec(x_14); +x_24 = 1; +x_25 = lean_usize_sub(x_23, x_24); +x_26 = lean_usize_land(x_22, x_25); +x_27 = lean_array_uget(x_13, x_26); +x_28 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__15(x_6, x_27); +if (x_28 == 0) +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; +x_29 = lean_unsigned_to_nat(1u); +x_30 = lean_nat_add(x_12, x_29); +lean_dec(x_12); +lean_ctor_set(x_4, 2, x_27); +lean_ctor_set(x_4, 1, x_10); +x_31 = lean_array_uset(x_13, x_26, x_4); +x_32 = lean_unsigned_to_nat(4u); +x_33 = lean_nat_mul(x_30, x_32); +x_34 = lean_unsigned_to_nat(3u); +x_35 = lean_nat_div(x_33, x_34); +lean_dec(x_33); +x_36 = lean_array_get_size(x_31); +x_37 = lean_nat_dec_le(x_35, x_36); +lean_dec(x_36); +lean_dec(x_35); +if (x_37 == 0) +{ +lean_object* x_38; +x_38 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__16(x_31); +lean_ctor_set(x_3, 1, x_38); +lean_ctor_set(x_3, 0, x_30); +x_4 = x_8; +goto _start; +} +else +{ +lean_ctor_set(x_3, 1, x_31); +lean_ctor_set(x_3, 0, x_30); +x_4 = x_8; +goto _start; +} +} +else +{ +lean_object* x_41; lean_object* x_42; lean_object* x_43; +lean_free_object(x_4); +lean_inc(x_1); +x_41 = lean_array_uset(x_13, x_26, x_1); +x_42 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__19(x_6, x_10, x_27); +x_43 = lean_array_uset(x_41, x_26, x_42); +lean_ctor_set(x_3, 1, x_43); +x_4 = x_8; +goto _start; +} +} +else +{ +lean_object* x_45; lean_object* x_46; lean_object* x_47; uint64_t x_48; uint64_t x_49; uint64_t x_50; uint64_t x_51; uint64_t x_52; uint64_t x_53; uint64_t x_54; size_t x_55; size_t x_56; size_t x_57; size_t x_58; size_t x_59; lean_object* x_60; uint8_t x_61; +x_45 = lean_ctor_get(x_3, 0); +x_46 = lean_ctor_get(x_3, 1); +lean_inc(x_46); +lean_inc(x_45); +lean_dec(x_3); +x_47 = lean_array_get_size(x_46); +x_48 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_6); +x_49 = 32; +x_50 = lean_uint64_shift_right(x_48, x_49); +x_51 = lean_uint64_xor(x_48, x_50); +x_52 = 16; +x_53 = lean_uint64_shift_right(x_51, x_52); +x_54 = lean_uint64_xor(x_51, x_53); +x_55 = lean_uint64_to_usize(x_54); +x_56 = lean_usize_of_nat(x_47); +lean_dec(x_47); +x_57 = 1; +x_58 = lean_usize_sub(x_56, x_57); +x_59 = lean_usize_land(x_55, x_58); +x_60 = lean_array_uget(x_46, x_59); +x_61 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__15(x_6, x_60); +if (x_61 == 0) +{ +lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; uint8_t x_70; +x_62 = lean_unsigned_to_nat(1u); +x_63 = lean_nat_add(x_45, x_62); +lean_dec(x_45); +lean_ctor_set(x_4, 2, x_60); +lean_ctor_set(x_4, 1, x_10); +x_64 = lean_array_uset(x_46, x_59, x_4); +x_65 = lean_unsigned_to_nat(4u); +x_66 = lean_nat_mul(x_63, x_65); +x_67 = lean_unsigned_to_nat(3u); +x_68 = lean_nat_div(x_66, x_67); +lean_dec(x_66); +x_69 = lean_array_get_size(x_64); +x_70 = lean_nat_dec_le(x_68, x_69); +lean_dec(x_69); +lean_dec(x_68); +if (x_70 == 0) +{ +lean_object* x_71; lean_object* x_72; +x_71 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__16(x_64); +x_72 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_72, 0, x_63); +lean_ctor_set(x_72, 1, x_71); +x_3 = x_72; +x_4 = x_8; +goto _start; +} +else +{ +lean_object* x_74; +x_74 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_74, 0, x_63); +lean_ctor_set(x_74, 1, x_64); +x_3 = x_74; +x_4 = x_8; +goto _start; +} +} +else +{ +lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; +lean_free_object(x_4); +lean_inc(x_1); +x_76 = lean_array_uset(x_46, x_59, x_1); +x_77 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__19(x_6, x_10, x_60); +x_78 = lean_array_uset(x_76, x_59, x_77); +x_79 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_79, 0, x_45); +lean_ctor_set(x_79, 1, x_78); +x_3 = x_79; +x_4 = x_8; +goto _start; +} +} +} +else +{ +lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; uint64_t x_90; uint64_t x_91; uint64_t x_92; uint64_t x_93; uint64_t x_94; uint64_t x_95; uint64_t x_96; size_t x_97; size_t x_98; size_t x_99; size_t x_100; size_t x_101; lean_object* x_102; uint8_t x_103; +x_81 = lean_ctor_get(x_4, 0); +x_82 = lean_ctor_get(x_4, 1); +x_83 = lean_ctor_get(x_4, 2); +lean_inc(x_83); +lean_inc(x_82); +lean_inc(x_81); +lean_dec(x_4); +x_84 = lean_ctor_get(x_2, 3); +x_85 = l_Lean_Linter_UnusedVariables_followAliases(x_84, x_82); +x_86 = lean_ctor_get(x_3, 0); +lean_inc(x_86); +x_87 = lean_ctor_get(x_3, 1); +lean_inc(x_87); +if (lean_is_exclusive(x_3)) { + lean_ctor_release(x_3, 0); + lean_ctor_release(x_3, 1); + x_88 = x_3; +} else { + lean_dec_ref(x_3); + x_88 = lean_box(0); +} +x_89 = lean_array_get_size(x_87); +x_90 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_81); +x_91 = 32; +x_92 = lean_uint64_shift_right(x_90, x_91); +x_93 = lean_uint64_xor(x_90, x_92); +x_94 = 16; +x_95 = lean_uint64_shift_right(x_93, x_94); +x_96 = lean_uint64_xor(x_93, x_95); +x_97 = lean_uint64_to_usize(x_96); +x_98 = lean_usize_of_nat(x_89); +lean_dec(x_89); +x_99 = 1; +x_100 = lean_usize_sub(x_98, x_99); +x_101 = lean_usize_land(x_97, x_100); +x_102 = lean_array_uget(x_87, x_101); +x_103 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__15(x_81, x_102); +if (x_103 == 0) +{ +lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; uint8_t x_113; +x_104 = lean_unsigned_to_nat(1u); +x_105 = lean_nat_add(x_86, x_104); +lean_dec(x_86); +x_106 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_106, 0, x_81); +lean_ctor_set(x_106, 1, x_85); +lean_ctor_set(x_106, 2, x_102); +x_107 = lean_array_uset(x_87, x_101, x_106); +x_108 = lean_unsigned_to_nat(4u); +x_109 = lean_nat_mul(x_105, x_108); +x_110 = lean_unsigned_to_nat(3u); +x_111 = lean_nat_div(x_109, x_110); +lean_dec(x_109); +x_112 = lean_array_get_size(x_107); +x_113 = lean_nat_dec_le(x_111, x_112); +lean_dec(x_112); +lean_dec(x_111); +if (x_113 == 0) +{ +lean_object* x_114; lean_object* x_115; +x_114 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__16(x_107); +if (lean_is_scalar(x_88)) { + x_115 = lean_alloc_ctor(0, 2, 0); +} else { + x_115 = x_88; +} +lean_ctor_set(x_115, 0, x_105); +lean_ctor_set(x_115, 1, x_114); +x_3 = x_115; +x_4 = x_83; +goto _start; +} +else +{ +lean_object* x_117; +if (lean_is_scalar(x_88)) { + x_117 = lean_alloc_ctor(0, 2, 0); +} else { + x_117 = x_88; +} +lean_ctor_set(x_117, 0, x_105); +lean_ctor_set(x_117, 1, x_107); +x_3 = x_117; +x_4 = x_83; +goto _start; +} +} +else +{ +lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; +lean_inc(x_1); +x_119 = lean_array_uset(x_87, x_101, x_1); +x_120 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__19(x_81, x_85, x_102); +x_121 = lean_array_uset(x_119, x_101, x_120); +if (lean_is_scalar(x_88)) { + x_122 = lean_alloc_ctor(0, 2, 0); +} else { + x_122 = x_88; +} +lean_ctor_set(x_122, 0, x_86); +lean_ctor_set(x_122, 1, x_121); +x_3 = x_122; +x_4 = x_83; +goto _start; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__2(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +return x_1; +} +else +{ +uint8_t x_3; +x_3 = !lean_is_exclusive(x_2); +if (x_3 == 0) +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; uint64_t x_10; uint64_t x_11; uint64_t x_12; uint64_t x_13; uint64_t x_14; uint64_t x_15; uint64_t x_16; size_t x_17; size_t x_18; size_t x_19; size_t x_20; size_t x_21; lean_object* x_22; uint8_t x_23; +x_4 = lean_ctor_get(x_2, 0); +x_5 = lean_ctor_get(x_2, 1); +x_6 = lean_ctor_get(x_2, 2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_1, 1); +lean_inc(x_8); +x_9 = lean_array_get_size(x_8); +x_10 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_4); +x_11 = 32; +x_12 = lean_uint64_shift_right(x_10, x_11); +x_13 = lean_uint64_xor(x_10, x_12); +x_14 = 16; +x_15 = lean_uint64_shift_right(x_13, x_14); +x_16 = lean_uint64_xor(x_13, x_15); +x_17 = lean_uint64_to_usize(x_16); +x_18 = lean_usize_of_nat(x_9); +lean_dec(x_9); +x_19 = 1; +x_20 = lean_usize_sub(x_18, x_19); +x_21 = lean_usize_land(x_17, x_20); +x_22 = lean_array_uget(x_8, x_21); +x_23 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_4, x_22); +lean_dec(x_22); +lean_dec(x_4); +if (x_23 == 0) +{ +lean_dec(x_8); +lean_dec(x_7); +lean_free_object(x_2); +lean_dec(x_5); +x_2 = x_6; +goto _start; +} +else +{ +uint8_t x_25; +x_25 = !lean_is_exclusive(x_1); +if (x_25 == 0) +{ +lean_object* x_26; lean_object* x_27; uint64_t x_28; uint64_t x_29; uint64_t x_30; uint64_t x_31; uint64_t x_32; size_t x_33; size_t x_34; lean_object* x_35; uint8_t x_36; +x_26 = lean_ctor_get(x_1, 1); +lean_dec(x_26); +x_27 = lean_ctor_get(x_1, 0); +lean_dec(x_27); +x_28 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_5); +x_29 = lean_uint64_shift_right(x_28, x_11); +x_30 = lean_uint64_xor(x_28, x_29); +x_31 = lean_uint64_shift_right(x_30, x_14); +x_32 = lean_uint64_xor(x_30, x_31); +x_33 = lean_uint64_to_usize(x_32); +x_34 = lean_usize_land(x_33, x_20); +x_35 = lean_array_uget(x_8, x_34); +x_36 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_5, x_35); +if (x_36 == 0) +{ +lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; uint8_t x_46; +x_37 = lean_unsigned_to_nat(1u); +x_38 = lean_nat_add(x_7, x_37); +lean_dec(x_7); +x_39 = lean_box(0); +lean_ctor_set(x_2, 2, x_35); +lean_ctor_set(x_2, 1, x_39); +lean_ctor_set(x_2, 0, x_5); +x_40 = lean_array_uset(x_8, x_34, x_2); +x_41 = lean_unsigned_to_nat(4u); +x_42 = lean_nat_mul(x_38, x_41); +x_43 = lean_unsigned_to_nat(3u); +x_44 = lean_nat_div(x_42, x_43); +lean_dec(x_42); +x_45 = lean_array_get_size(x_40); +x_46 = lean_nat_dec_le(x_44, x_45); +lean_dec(x_45); +lean_dec(x_44); +if (x_46 == 0) +{ +lean_object* x_47; +x_47 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_40); +lean_ctor_set(x_1, 1, x_47); +lean_ctor_set(x_1, 0, x_38); +x_2 = x_6; +goto _start; +} +else +{ +lean_ctor_set(x_1, 1, x_40); +lean_ctor_set(x_1, 0, x_38); +x_2 = x_6; +goto _start; +} +} +else +{ +lean_dec(x_35); +lean_free_object(x_2); +lean_dec(x_5); +x_2 = x_6; +goto _start; +} +} +else +{ +uint64_t x_51; uint64_t x_52; uint64_t x_53; uint64_t x_54; uint64_t x_55; size_t x_56; size_t x_57; lean_object* x_58; uint8_t x_59; +lean_dec(x_1); +x_51 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_5); +x_52 = lean_uint64_shift_right(x_51, x_11); +x_53 = lean_uint64_xor(x_51, x_52); +x_54 = lean_uint64_shift_right(x_53, x_14); +x_55 = lean_uint64_xor(x_53, x_54); +x_56 = lean_uint64_to_usize(x_55); +x_57 = lean_usize_land(x_56, x_20); +x_58 = lean_array_uget(x_8, x_57); +x_59 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_5, x_58); +if (x_59 == 0) +{ +lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; uint8_t x_69; +x_60 = lean_unsigned_to_nat(1u); +x_61 = lean_nat_add(x_7, x_60); +lean_dec(x_7); +x_62 = lean_box(0); +lean_ctor_set(x_2, 2, x_58); +lean_ctor_set(x_2, 1, x_62); +lean_ctor_set(x_2, 0, x_5); +x_63 = lean_array_uset(x_8, x_57, x_2); +x_64 = lean_unsigned_to_nat(4u); +x_65 = lean_nat_mul(x_61, x_64); +x_66 = lean_unsigned_to_nat(3u); +x_67 = lean_nat_div(x_65, x_66); +lean_dec(x_65); +x_68 = lean_array_get_size(x_63); +x_69 = lean_nat_dec_le(x_67, x_68); +lean_dec(x_68); +lean_dec(x_67); +if (x_69 == 0) +{ +lean_object* x_70; lean_object* x_71; +x_70 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_63); +x_71 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_71, 0, x_61); +lean_ctor_set(x_71, 1, x_70); +x_1 = x_71; +x_2 = x_6; +goto _start; +} +else +{ +lean_object* x_73; +x_73 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_73, 0, x_61); +lean_ctor_set(x_73, 1, x_63); +x_1 = x_73; +x_2 = x_6; +goto _start; +} +} +else +{ +lean_object* x_75; +lean_dec(x_58); +lean_free_object(x_2); +lean_dec(x_5); +x_75 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_75, 0, x_7); +lean_ctor_set(x_75, 1, x_8); +x_1 = x_75; +x_2 = x_6; +goto _start; +} +} +} +} +else +{ +lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; uint64_t x_83; uint64_t x_84; uint64_t x_85; uint64_t x_86; uint64_t x_87; uint64_t x_88; uint64_t x_89; size_t x_90; size_t x_91; size_t x_92; size_t x_93; size_t x_94; lean_object* x_95; uint8_t x_96; +x_77 = lean_ctor_get(x_2, 0); x_78 = lean_ctor_get(x_2, 1); x_79 = lean_ctor_get(x_2, 2); lean_inc(x_79); lean_inc(x_78); lean_inc(x_77); lean_dec(x_2); -x_80 = lean_ctor_get(x_1, 0); -lean_inc(x_80); -x_81 = lean_ctor_get(x_1, 1); -lean_inc(x_81); -x_82 = lean_array_get_size(x_81); -x_83 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_77); -x_84 = 32; -x_85 = lean_uint64_shift_right(x_83, x_84); -x_86 = lean_uint64_xor(x_83, x_85); -x_87 = 16; -x_88 = lean_uint64_shift_right(x_86, x_87); -x_89 = lean_uint64_xor(x_86, x_88); -x_90 = lean_uint64_to_usize(x_89); -x_91 = lean_usize_of_nat(x_82); -lean_dec(x_82); -x_92 = 1; -x_93 = lean_usize_sub(x_91, x_92); -x_94 = lean_usize_land(x_90, x_93); -x_95 = lean_array_uget(x_81, x_94); -x_96 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_77, x_95); -lean_dec(x_95); -lean_dec(x_77); -if (x_96 == 0) +x_80 = lean_ctor_get(x_1, 0); +lean_inc(x_80); +x_81 = lean_ctor_get(x_1, 1); +lean_inc(x_81); +x_82 = lean_array_get_size(x_81); +x_83 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_77); +x_84 = 32; +x_85 = lean_uint64_shift_right(x_83, x_84); +x_86 = lean_uint64_xor(x_83, x_85); +x_87 = 16; +x_88 = lean_uint64_shift_right(x_86, x_87); +x_89 = lean_uint64_xor(x_86, x_88); +x_90 = lean_uint64_to_usize(x_89); +x_91 = lean_usize_of_nat(x_82); +lean_dec(x_82); +x_92 = 1; +x_93 = lean_usize_sub(x_91, x_92); +x_94 = lean_usize_land(x_90, x_93); +x_95 = lean_array_uget(x_81, x_94); +x_96 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_77, x_95); +lean_dec(x_95); +lean_dec(x_77); +if (x_96 == 0) +{ +lean_dec(x_81); +lean_dec(x_80); +lean_dec(x_78); +x_2 = x_79; +goto _start; +} +else +{ +lean_object* x_98; uint64_t x_99; uint64_t x_100; uint64_t x_101; uint64_t x_102; uint64_t x_103; size_t x_104; size_t x_105; lean_object* x_106; uint8_t x_107; +if (lean_is_exclusive(x_1)) { + lean_ctor_release(x_1, 0); + lean_ctor_release(x_1, 1); + x_98 = x_1; +} else { + lean_dec_ref(x_1); + x_98 = lean_box(0); +} +x_99 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_78); +x_100 = lean_uint64_shift_right(x_99, x_84); +x_101 = lean_uint64_xor(x_99, x_100); +x_102 = lean_uint64_shift_right(x_101, x_87); +x_103 = lean_uint64_xor(x_101, x_102); +x_104 = lean_uint64_to_usize(x_103); +x_105 = lean_usize_land(x_104, x_93); +x_106 = lean_array_uget(x_81, x_105); +x_107 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_78, x_106); +if (x_107 == 0) +{ +lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; uint8_t x_118; +x_108 = lean_unsigned_to_nat(1u); +x_109 = lean_nat_add(x_80, x_108); +lean_dec(x_80); +x_110 = lean_box(0); +x_111 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_111, 0, x_78); +lean_ctor_set(x_111, 1, x_110); +lean_ctor_set(x_111, 2, x_106); +x_112 = lean_array_uset(x_81, x_105, x_111); +x_113 = lean_unsigned_to_nat(4u); +x_114 = lean_nat_mul(x_109, x_113); +x_115 = lean_unsigned_to_nat(3u); +x_116 = lean_nat_div(x_114, x_115); +lean_dec(x_114); +x_117 = lean_array_get_size(x_112); +x_118 = lean_nat_dec_le(x_116, x_117); +lean_dec(x_117); +lean_dec(x_116); +if (x_118 == 0) +{ +lean_object* x_119; lean_object* x_120; +x_119 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_112); +if (lean_is_scalar(x_98)) { + x_120 = lean_alloc_ctor(0, 2, 0); +} else { + x_120 = x_98; +} +lean_ctor_set(x_120, 0, x_109); +lean_ctor_set(x_120, 1, x_119); +x_1 = x_120; +x_2 = x_79; +goto _start; +} +else +{ +lean_object* x_122; +if (lean_is_scalar(x_98)) { + x_122 = lean_alloc_ctor(0, 2, 0); +} else { + x_122 = x_98; +} +lean_ctor_set(x_122, 0, x_109); +lean_ctor_set(x_122, 1, x_112); +x_1 = x_122; +x_2 = x_79; +goto _start; +} +} +else +{ +lean_object* x_124; +lean_dec(x_106); +lean_dec(x_78); +if (lean_is_scalar(x_98)) { + x_124 = lean_alloc_ctor(0, 2, 0); +} else { + x_124 = x_98; +} +lean_ctor_set(x_124, 0, x_80); +lean_ctor_set(x_124, 1, x_81); +x_1 = x_124; +x_2 = x_79; +goto _start; +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +if (lean_obj_tag(x_3) == 0) +{ +lean_inc(x_2); +return x_2; +} +else +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; uint8_t x_7; +x_4 = lean_ctor_get(x_3, 0); +x_5 = lean_ctor_get(x_3, 1); +x_6 = lean_ctor_get(x_3, 2); +x_7 = lean_name_eq(x_4, x_1); +if (x_7 == 0) +{ +x_3 = x_6; +goto _start; +} +else +{ +lean_inc(x_5); +return x_5; +} +} +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__4(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +return x_1; +} +else +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_3 = lean_ctor_get(x_2, 0); +x_4 = lean_ctor_get(x_2, 1); +x_5 = lean_ctor_get(x_2, 2); +lean_inc(x_4); +lean_inc(x_3); +x_6 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_6, 0, x_3); +lean_ctor_set(x_6, 1, x_4); +x_7 = lean_array_push(x_1, x_6); +x_1 = x_7; +x_2 = x_5; +goto _start; +} +} +} +static lean_object* _init_l_panic___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__8___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Command_instMonadCommandElabM; +x_3 = l_instInhabitedOfMonad___rarg(x_2, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_panic___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_5 = l_panic___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__8___closed__1; +x_6 = lean_panic_fn(x_5, x_1); +x_7 = lean_apply_3(x_6, x_2, x_3, x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +if (lean_obj_tag(x_4) == 0) +{ +lean_object* x_9; lean_object* x_10; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_9 = l_List_reverse___rarg(x_5); +x_10 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set(x_10, 1, x_8); +return x_10; +} +else +{ +uint8_t x_11; +x_11 = !lean_is_exclusive(x_4); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_4, 0); +x_13 = lean_ctor_get(x_4, 1); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__7(x_1, x_2, x_3, x_12, x_6, x_7, x_8); +if (lean_obj_tag(x_14) == 0) +{ +lean_object* x_15; lean_object* x_16; +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); +lean_ctor_set(x_4, 1, x_5); +lean_ctor_set(x_4, 0, x_15); +{ +lean_object* _tmp_3 = x_13; +lean_object* _tmp_4 = x_4; +lean_object* _tmp_7 = x_16; +x_4 = _tmp_3; +x_5 = _tmp_4; +x_8 = _tmp_7; +} +goto _start; +} +else +{ +uint8_t x_18; +lean_free_object(x_4); +lean_dec(x_13); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_18 = !lean_is_exclusive(x_14); +if (x_18 == 0) { -lean_dec(x_81); -lean_dec(x_80); -lean_dec(x_78); -x_2 = x_79; +return x_14; +} +else +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_14, 0); +x_20 = lean_ctor_get(x_14, 1); +lean_inc(x_20); +lean_inc(x_19); +lean_dec(x_14); +x_21 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_21, 0, x_19); +lean_ctor_set(x_21, 1, x_20); +return x_21; +} +} +} +else +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_4, 0); +x_23 = lean_ctor_get(x_4, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_4); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_24 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__7(x_1, x_2, x_3, x_22, x_6, x_7, x_8); +if (lean_obj_tag(x_24) == 0) +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_24, 0); +lean_inc(x_25); +x_26 = lean_ctor_get(x_24, 1); +lean_inc(x_26); +lean_dec(x_24); +x_27 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_5); +x_4 = x_23; +x_5 = x_27; +x_8 = x_26; goto _start; } else { -lean_object* x_98; uint64_t x_99; uint64_t x_100; uint64_t x_101; uint64_t x_102; uint64_t x_103; size_t x_104; size_t x_105; lean_object* x_106; uint8_t x_107; -if (lean_is_exclusive(x_1)) { - lean_ctor_release(x_1, 0); - lean_ctor_release(x_1, 1); - x_98 = x_1; +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +lean_dec(x_23); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_29 = lean_ctor_get(x_24, 0); +lean_inc(x_29); +x_30 = lean_ctor_get(x_24, 1); +lean_inc(x_30); +if (lean_is_exclusive(x_24)) { + lean_ctor_release(x_24, 0); + lean_ctor_release(x_24, 1); + x_31 = x_24; } else { - lean_dec_ref(x_1); - x_98 = lean_box(0); + lean_dec_ref(x_24); + x_31 = lean_box(0); } -x_99 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_78); -x_100 = lean_uint64_shift_right(x_99, x_84); -x_101 = lean_uint64_xor(x_99, x_100); -x_102 = lean_uint64_shift_right(x_101, x_87); -x_103 = lean_uint64_xor(x_101, x_102); -x_104 = lean_uint64_to_usize(x_103); -x_105 = lean_usize_land(x_104, x_93); -x_106 = lean_array_uget(x_81, x_105); -x_107 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_78, x_106); -if (x_107 == 0) +if (lean_is_scalar(x_31)) { + x_32 = lean_alloc_ctor(1, 2, 0); +} else { + x_32 = x_31; +} +lean_ctor_set(x_32, 0, x_29); +lean_ctor_set(x_32, 1, x_30); +return x_32; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: { -lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; uint8_t x_118; -x_108 = lean_unsigned_to_nat(1u); -x_109 = lean_nat_add(x_80, x_108); -lean_dec(x_80); -x_110 = lean_box(0); -x_111 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_111, 0, x_78); -lean_ctor_set(x_111, 1, x_110); -lean_ctor_set(x_111, 2, x_106); -x_112 = lean_array_uset(x_81, x_105, x_111); -x_113 = lean_unsigned_to_nat(4u); -x_114 = lean_nat_mul(x_109, x_113); -x_115 = lean_unsigned_to_nat(3u); -x_116 = lean_nat_div(x_114, x_115); -lean_dec(x_114); -x_117 = lean_array_get_size(x_112); -x_118 = lean_nat_dec_le(x_116, x_117); -lean_dec(x_117); -lean_dec(x_116); -if (x_118 == 0) +if (lean_obj_tag(x_3) == 0) { -lean_object* x_119; lean_object* x_120; -x_119 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_112); -if (lean_is_scalar(x_98)) { - x_120 = lean_alloc_ctor(0, 2, 0); -} else { - x_120 = x_98; +switch (lean_obj_tag(x_4)) { +case 0: +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_8 = lean_ctor_get(x_4, 0); +lean_inc(x_8); +x_9 = lean_ctor_get(x_4, 1); +lean_inc(x_9); +lean_dec(x_4); +x_10 = l_Lean_Elab_PartialContextInfo_mergeIntoOuter_x3f(x_8, x_3); +x_3 = x_10; +x_4 = x_9; +goto _start; +} +case 1: +{ +lean_object* x_12; lean_object* x_13; +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_12 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__4; +x_13 = l_panic___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__8(x_12, x_5, x_6, x_7); +return x_13; +} +default: +{ +lean_object* x_14; lean_object* x_15; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_14 = lean_box(0); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_7); +return x_15; +} +} +} +else +{ +switch (lean_obj_tag(x_4)) { +case 0: +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_4, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_4, 1); +lean_inc(x_17); +lean_dec(x_4); +x_18 = l_Lean_Elab_PartialContextInfo_mergeIntoOuter_x3f(x_16, x_3); +x_3 = x_18; +x_4 = x_17; +goto _start; +} +case 1: +{ +uint8_t x_20; +x_20 = !lean_is_exclusive(x_3); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_21 = lean_ctor_get(x_3, 0); +x_22 = lean_ctor_get(x_4, 0); +lean_inc(x_22); +x_23 = lean_ctor_get(x_4, 1); +lean_inc(x_23); +lean_dec(x_4); +lean_inc(x_1); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_23); +lean_inc(x_22); +lean_inc(x_21); +x_24 = lean_apply_6(x_1, x_21, x_22, x_23, x_5, x_6, x_7); +if (lean_obj_tag(x_24) == 0) +{ +lean_object* x_25; uint8_t x_26; +x_25 = lean_ctor_get(x_24, 0); +lean_inc(x_25); +x_26 = lean_unbox(x_25); +lean_dec(x_25); +if (x_26 == 0) +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; +lean_dec(x_1); +x_27 = lean_ctor_get(x_24, 1); +lean_inc(x_27); +lean_dec(x_24); +x_28 = lean_box(0); +x_29 = lean_apply_7(x_2, x_21, x_22, x_23, x_28, x_5, x_6, x_27); +if (lean_obj_tag(x_29) == 0) +{ +uint8_t x_30; +x_30 = !lean_is_exclusive(x_29); +if (x_30 == 0) +{ +lean_object* x_31; +x_31 = lean_ctor_get(x_29, 0); +lean_ctor_set(x_3, 0, x_31); +lean_ctor_set(x_29, 0, x_3); +return x_29; +} +else +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_29, 0); +x_33 = lean_ctor_get(x_29, 1); +lean_inc(x_33); +lean_inc(x_32); +lean_dec(x_29); +lean_ctor_set(x_3, 0, x_32); +x_34 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_34, 0, x_3); +lean_ctor_set(x_34, 1, x_33); +return x_34; } -lean_ctor_set(x_120, 0, x_109); -lean_ctor_set(x_120, 1, x_119); -x_1 = x_120; -x_2 = x_79; -goto _start; } else { -lean_object* x_122; -if (lean_is_scalar(x_98)) { - x_122 = lean_alloc_ctor(0, 2, 0); -} else { - x_122 = x_98; +uint8_t x_35; +lean_free_object(x_3); +x_35 = !lean_is_exclusive(x_29); +if (x_35 == 0) +{ +return x_29; +} +else +{ +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_29, 0); +x_37 = lean_ctor_get(x_29, 1); +lean_inc(x_37); +lean_inc(x_36); +lean_dec(x_29); +x_38 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_38, 0, x_36); +lean_ctor_set(x_38, 1, x_37); +return x_38; } -lean_ctor_set(x_122, 0, x_109); -lean_ctor_set(x_122, 1, x_112); -x_1 = x_122; -x_2 = x_79; -goto _start; } } else { -lean_object* x_124; -lean_dec(x_106); -lean_dec(x_78); -if (lean_is_scalar(x_98)) { - x_124 = lean_alloc_ctor(0, 2, 0); -} else { - x_124 = x_98; +lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_39 = lean_ctor_get(x_24, 1); +lean_inc(x_39); +lean_dec(x_24); +lean_inc(x_21); +x_40 = l_Lean_Elab_Info_updateContext_x3f(x_3, x_22); +x_41 = l_Lean_PersistentArray_toList___rarg(x_23); +x_42 = lean_box(0); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_2); +x_43 = l_List_mapM_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__9(x_1, x_2, x_40, x_41, x_42, x_5, x_6, x_39); +if (lean_obj_tag(x_43) == 0) +{ +lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_44 = lean_ctor_get(x_43, 0); +lean_inc(x_44); +x_45 = lean_ctor_get(x_43, 1); +lean_inc(x_45); +lean_dec(x_43); +x_46 = lean_apply_7(x_2, x_21, x_22, x_23, x_44, x_5, x_6, x_45); +if (lean_obj_tag(x_46) == 0) +{ +uint8_t x_47; +x_47 = !lean_is_exclusive(x_46); +if (x_47 == 0) +{ +lean_object* x_48; lean_object* x_49; +x_48 = lean_ctor_get(x_46, 0); +x_49 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_49, 0, x_48); +lean_ctor_set(x_46, 0, x_49); +return x_46; } -lean_ctor_set(x_124, 0, x_80); -lean_ctor_set(x_124, 1, x_81); -x_1 = x_124; -x_2 = x_79; -goto _start; +else +{ +lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_50 = lean_ctor_get(x_46, 0); +x_51 = lean_ctor_get(x_46, 1); +lean_inc(x_51); +lean_inc(x_50); +lean_dec(x_46); +x_52 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_52, 0, x_50); +x_53 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_53, 0, x_52); +lean_ctor_set(x_53, 1, x_51); +return x_53; } } +else +{ +uint8_t x_54; +x_54 = !lean_is_exclusive(x_46); +if (x_54 == 0) +{ +return x_46; } +else +{ +lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_55 = lean_ctor_get(x_46, 0); +x_56 = lean_ctor_get(x_46, 1); +lean_inc(x_56); +lean_inc(x_55); +lean_dec(x_46); +x_57 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_57, 0, x_55); +lean_ctor_set(x_57, 1, x_56); +return x_57; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__3(lean_object* x_1, lean_object* x_2) { -_start: +else { -if (lean_obj_tag(x_2) == 0) +uint8_t x_58; +lean_dec(x_23); +lean_dec(x_22); +lean_dec(x_21); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +x_58 = !lean_is_exclusive(x_43); +if (x_58 == 0) { -return x_1; +return x_43; } else { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_3 = lean_ctor_get(x_2, 0); -x_4 = lean_ctor_get(x_2, 1); -x_5 = lean_ctor_get(x_2, 2); -lean_inc(x_4); -lean_inc(x_3); -x_6 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_6, 0, x_3); -lean_ctor_set(x_6, 1, x_4); -x_7 = lean_array_push(x_1, x_6); -x_1 = x_7; -x_2 = x_5; -goto _start; +lean_object* x_59; lean_object* x_60; lean_object* x_61; +x_59 = lean_ctor_get(x_43, 0); +x_60 = lean_ctor_get(x_43, 1); +lean_inc(x_60); +lean_inc(x_59); +lean_dec(x_43); +x_61 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_61, 0, x_59); +lean_ctor_set(x_61, 1, x_60); +return x_61; } } } -static lean_object* _init_l_panic___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__8___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Command_instMonadCommandElabM; -x_3 = l_instInhabitedOfMonad___rarg(x_2, x_1); -return x_3; } +else +{ +uint8_t x_62; +lean_dec(x_23); +lean_dec(x_22); +lean_free_object(x_3); +lean_dec(x_21); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +lean_dec(x_1); +x_62 = !lean_is_exclusive(x_24); +if (x_62 == 0) +{ +return x_24; } -LEAN_EXPORT lean_object* l_panic___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: +else { -lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_5 = l_panic___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__8___closed__1; -x_6 = lean_panic_fn(x_5, x_1); -x_7 = lean_apply_3(x_6, x_2, x_3, x_4); -return x_7; +lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_63 = lean_ctor_get(x_24, 0); +x_64 = lean_ctor_get(x_24, 1); +lean_inc(x_64); +lean_inc(x_63); +lean_dec(x_24); +x_65 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_65, 0, x_63); +lean_ctor_set(x_65, 1, x_64); +return x_65; } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -if (lean_obj_tag(x_4) == 0) +} +else { -lean_object* x_9; lean_object* x_10; -lean_dec(x_7); -lean_dec(x_6); +lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; +x_66 = lean_ctor_get(x_3, 0); +lean_inc(x_66); lean_dec(x_3); -lean_dec(x_2); +x_67 = lean_ctor_get(x_4, 0); +lean_inc(x_67); +x_68 = lean_ctor_get(x_4, 1); +lean_inc(x_68); +lean_dec(x_4); +lean_inc(x_1); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_68); +lean_inc(x_67); +lean_inc(x_66); +x_69 = lean_apply_6(x_1, x_66, x_67, x_68, x_5, x_6, x_7); +if (lean_obj_tag(x_69) == 0) +{ +lean_object* x_70; uint8_t x_71; +x_70 = lean_ctor_get(x_69, 0); +lean_inc(x_70); +x_71 = lean_unbox(x_70); +lean_dec(x_70); +if (x_71 == 0) +{ +lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_dec(x_1); -x_9 = l_List_reverse___rarg(x_5); -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_9); -lean_ctor_set(x_10, 1, x_8); -return x_10; +x_72 = lean_ctor_get(x_69, 1); +lean_inc(x_72); +lean_dec(x_69); +x_73 = lean_box(0); +x_74 = lean_apply_7(x_2, x_66, x_67, x_68, x_73, x_5, x_6, x_72); +if (lean_obj_tag(x_74) == 0) +{ +lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; +x_75 = lean_ctor_get(x_74, 0); +lean_inc(x_75); +x_76 = lean_ctor_get(x_74, 1); +lean_inc(x_76); +if (lean_is_exclusive(x_74)) { + lean_ctor_release(x_74, 0); + lean_ctor_release(x_74, 1); + x_77 = x_74; +} else { + lean_dec_ref(x_74); + x_77 = lean_box(0); +} +x_78 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_78, 0, x_75); +if (lean_is_scalar(x_77)) { + x_79 = lean_alloc_ctor(0, 2, 0); +} else { + x_79 = x_77; +} +lean_ctor_set(x_79, 0, x_78); +lean_ctor_set(x_79, 1, x_76); +return x_79; } else { -uint8_t x_11; -x_11 = !lean_is_exclusive(x_4); -if (x_11 == 0) +lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; +x_80 = lean_ctor_get(x_74, 0); +lean_inc(x_80); +x_81 = lean_ctor_get(x_74, 1); +lean_inc(x_81); +if (lean_is_exclusive(x_74)) { + lean_ctor_release(x_74, 0); + lean_ctor_release(x_74, 1); + x_82 = x_74; +} else { + lean_dec_ref(x_74); + x_82 = lean_box(0); +} +if (lean_is_scalar(x_82)) { + x_83 = lean_alloc_ctor(1, 2, 0); +} else { + x_83 = x_82; +} +lean_ctor_set(x_83, 0, x_80); +lean_ctor_set(x_83, 1, x_81); +return x_83; +} +} +else { -lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_12 = lean_ctor_get(x_4, 0); -x_13 = lean_ctor_get(x_4, 1); -lean_inc(x_7); +lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; +x_84 = lean_ctor_get(x_69, 1); +lean_inc(x_84); +lean_dec(x_69); +lean_inc(x_66); +x_85 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_85, 0, x_66); +x_86 = l_Lean_Elab_Info_updateContext_x3f(x_85, x_67); +x_87 = l_Lean_PersistentArray_toList___rarg(x_68); +x_88 = lean_box(0); lean_inc(x_6); -lean_inc(x_3); +lean_inc(x_5); lean_inc(x_2); -lean_inc(x_1); -x_14 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__7(x_1, x_2, x_3, x_12, x_6, x_7, x_8); -if (lean_obj_tag(x_14) == 0) +x_89 = l_List_mapM_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__9(x_1, x_2, x_86, x_87, x_88, x_5, x_6, x_84); +if (lean_obj_tag(x_89) == 0) { -lean_object* x_15; lean_object* x_16; -x_15 = lean_ctor_get(x_14, 0); -lean_inc(x_15); -x_16 = lean_ctor_get(x_14, 1); -lean_inc(x_16); -lean_dec(x_14); -lean_ctor_set(x_4, 1, x_5); -lean_ctor_set(x_4, 0, x_15); +lean_object* x_90; lean_object* x_91; lean_object* x_92; +x_90 = lean_ctor_get(x_89, 0); +lean_inc(x_90); +x_91 = lean_ctor_get(x_89, 1); +lean_inc(x_91); +lean_dec(x_89); +x_92 = lean_apply_7(x_2, x_66, x_67, x_68, x_90, x_5, x_6, x_91); +if (lean_obj_tag(x_92) == 0) +{ +lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; +x_93 = lean_ctor_get(x_92, 0); +lean_inc(x_93); +x_94 = lean_ctor_get(x_92, 1); +lean_inc(x_94); +if (lean_is_exclusive(x_92)) { + lean_ctor_release(x_92, 0); + lean_ctor_release(x_92, 1); + x_95 = x_92; +} else { + lean_dec_ref(x_92); + x_95 = lean_box(0); +} +x_96 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_96, 0, x_93); +if (lean_is_scalar(x_95)) { + x_97 = lean_alloc_ctor(0, 2, 0); +} else { + x_97 = x_95; +} +lean_ctor_set(x_97, 0, x_96); +lean_ctor_set(x_97, 1, x_94); +return x_97; +} +else { -lean_object* _tmp_3 = x_13; -lean_object* _tmp_4 = x_4; -lean_object* _tmp_7 = x_16; -x_4 = _tmp_3; -x_5 = _tmp_4; -x_8 = _tmp_7; +lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; +x_98 = lean_ctor_get(x_92, 0); +lean_inc(x_98); +x_99 = lean_ctor_get(x_92, 1); +lean_inc(x_99); +if (lean_is_exclusive(x_92)) { + lean_ctor_release(x_92, 0); + lean_ctor_release(x_92, 1); + x_100 = x_92; +} else { + lean_dec_ref(x_92); + x_100 = lean_box(0); +} +if (lean_is_scalar(x_100)) { + x_101 = lean_alloc_ctor(1, 2, 0); +} else { + x_101 = x_100; +} +lean_ctor_set(x_101, 0, x_98); +lean_ctor_set(x_101, 1, x_99); +return x_101; } -goto _start; } else { -uint8_t x_18; -lean_free_object(x_4); -lean_dec(x_13); -lean_dec(x_7); +lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; +lean_dec(x_68); +lean_dec(x_67); +lean_dec(x_66); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_18 = !lean_is_exclusive(x_14); -if (x_18 == 0) -{ -return x_14; +x_102 = lean_ctor_get(x_89, 0); +lean_inc(x_102); +x_103 = lean_ctor_get(x_89, 1); +lean_inc(x_103); +if (lean_is_exclusive(x_89)) { + lean_ctor_release(x_89, 0); + lean_ctor_release(x_89, 1); + x_104 = x_89; +} else { + lean_dec_ref(x_89); + x_104 = lean_box(0); } -else -{ -lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_19 = lean_ctor_get(x_14, 0); -x_20 = lean_ctor_get(x_14, 1); -lean_inc(x_20); -lean_inc(x_19); -lean_dec(x_14); -x_21 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_21, 0, x_19); -lean_ctor_set(x_21, 1, x_20); -return x_21; +if (lean_is_scalar(x_104)) { + x_105 = lean_alloc_ctor(1, 2, 0); +} else { + x_105 = x_104; } +lean_ctor_set(x_105, 0, x_102); +lean_ctor_set(x_105, 1, x_103); +return x_105; } } -else -{ -lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_22 = lean_ctor_get(x_4, 0); -x_23 = lean_ctor_get(x_4, 1); -lean_inc(x_23); -lean_inc(x_22); -lean_dec(x_4); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_3); -lean_inc(x_2); -lean_inc(x_1); -x_24 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__7(x_1, x_2, x_3, x_22, x_6, x_7, x_8); -if (lean_obj_tag(x_24) == 0) -{ -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_24, 0); -lean_inc(x_25); -x_26 = lean_ctor_get(x_24, 1); -lean_inc(x_26); -lean_dec(x_24); -x_27 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_5); -x_4 = x_23; -x_5 = x_27; -x_8 = x_26; -goto _start; } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; -lean_dec(x_23); -lean_dec(x_7); +lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; +lean_dec(x_68); +lean_dec(x_67); +lean_dec(x_66); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_29 = lean_ctor_get(x_24, 0); -lean_inc(x_29); -x_30 = lean_ctor_get(x_24, 1); -lean_inc(x_30); -if (lean_is_exclusive(x_24)) { - lean_ctor_release(x_24, 0); - lean_ctor_release(x_24, 1); - x_31 = x_24; +x_106 = lean_ctor_get(x_69, 0); +lean_inc(x_106); +x_107 = lean_ctor_get(x_69, 1); +lean_inc(x_107); +if (lean_is_exclusive(x_69)) { + lean_ctor_release(x_69, 0); + lean_ctor_release(x_69, 1); + x_108 = x_69; } else { - lean_dec_ref(x_24); - x_31 = lean_box(0); + lean_dec_ref(x_69); + x_108 = lean_box(0); } -if (lean_is_scalar(x_31)) { - x_32 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_108)) { + x_109 = lean_alloc_ctor(1, 2, 0); } else { - x_32 = x_31; -} -lean_ctor_set(x_32, 0, x_29); -lean_ctor_set(x_32, 1, x_30); -return x_32; -} -} -} + x_109 = x_108; } +lean_ctor_set(x_109, 0, x_106); +lean_ctor_set(x_109, 1, x_107); +return x_109; } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -if (lean_obj_tag(x_3) == 0) -{ -switch (lean_obj_tag(x_4)) { -case 0: -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; -x_8 = lean_ctor_get(x_4, 0); -lean_inc(x_8); -x_9 = lean_ctor_get(x_4, 1); -lean_inc(x_9); -lean_dec(x_4); -x_10 = l_Lean_Elab_PartialContextInfo_mergeIntoOuter_x3f(x_8, x_3); -x_3 = x_10; -x_4 = x_9; -goto _start; } -case 1: -{ -lean_object* x_12; lean_object* x_13; -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -x_12 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__4; -x_13 = l_panic___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__8(x_12, x_5, x_6, x_7); -return x_13; } default: { -lean_object* x_14; lean_object* x_15; +lean_object* x_110; lean_object* x_111; lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_14 = lean_box(0); -x_15 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_15, 0, x_14); -lean_ctor_set(x_15, 1, x_7); -return x_15; +x_110 = lean_box(0); +x_111 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_111, 0, x_110); +lean_ctor_set(x_111, 1, x_7); +return x_111; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +uint8_t x_7; lean_object* x_8; lean_object* x_9; +x_7 = 1; +x_8 = lean_box(x_7); +x_9 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_9, 0, x_8); +lean_ctor_set(x_9, 1, x_6); +return x_9; +} +} +static lean_object* _init_l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___lambda__2___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} } +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_9 = lean_box(0); +x_10 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379____closed__1; +x_11 = l_List_filterMapTR_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__1(x_5, x_10); +x_12 = l_List_filterMapTR_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__2(x_11, x_10); +if (lean_obj_tag(x_12) == 0) +{ +lean_object* x_13; uint8_t x_14; uint8_t x_15; +x_13 = lean_ctor_get(x_1, 0); +x_14 = 0; +x_15 = l_Lean_Elab_Info_contains(x_3, x_13, x_14); +if (x_15 == 0) +{ +lean_object* x_16; lean_object* x_17; +lean_dec(x_3); +x_16 = lean_box(0); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_16); +lean_ctor_set(x_17, 1, x_8); +return x_17; } +else +{ +lean_object* x_18; uint8_t x_19; uint8_t x_20; +x_18 = lean_ctor_get(x_1, 1); +x_19 = 1; +x_20 = l_Lean_Elab_Info_contains(x_3, x_18, x_19); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; +lean_dec(x_3); +x_21 = lean_box(0); +x_22 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_22, 0, x_21); +lean_ctor_set(x_22, 1, x_8); +return x_22; } else { -switch (lean_obj_tag(x_4)) { -case 0: +if (lean_obj_tag(x_3) == 3) { -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_4, 0); -lean_inc(x_16); -x_17 = lean_ctor_get(x_4, 1); -lean_inc(x_17); -lean_dec(x_4); -x_18 = l_Lean_Elab_PartialContextInfo_mergeIntoOuter_x3f(x_16, x_3); -x_3 = x_18; -x_4 = x_17; -goto _start; +uint8_t x_23; +x_23 = !lean_is_exclusive(x_3); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_3, 0); +x_25 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_25, 0, x_24); +lean_ctor_set(x_25, 1, x_9); +lean_ctor_set_tag(x_3, 1); +lean_ctor_set(x_3, 0, x_25); +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_3); +lean_ctor_set(x_26, 1, x_8); +return x_26; +} +else +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_27 = lean_ctor_get(x_3, 0); +lean_inc(x_27); +lean_dec(x_3); +x_28 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_9); +x_29 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_29, 0, x_28); +x_30 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_30, 0, x_29); +lean_ctor_set(x_30, 1, x_8); +return x_30; } -case 1: -{ -uint8_t x_20; -x_20 = !lean_is_exclusive(x_3); -if (x_20 == 0) -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_21 = lean_ctor_get(x_3, 0); -x_22 = lean_ctor_get(x_4, 0); -lean_inc(x_22); -x_23 = lean_ctor_get(x_4, 1); -lean_inc(x_23); -lean_dec(x_4); -lean_inc(x_1); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_23); -lean_inc(x_22); -lean_inc(x_21); -x_24 = lean_apply_6(x_1, x_21, x_22, x_23, x_5, x_6, x_7); -if (lean_obj_tag(x_24) == 0) +} +else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_25 = lean_ctor_get(x_24, 1); -lean_inc(x_25); -lean_dec(x_24); -lean_inc(x_21); -x_26 = l_Lean_Elab_Info_updateContext_x3f(x_3, x_22); -x_27 = l_Lean_PersistentArray_toList___rarg(x_23); -x_28 = lean_box(0); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_2); -x_29 = l_List_mapM_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__9(x_1, x_2, x_26, x_27, x_28, x_5, x_6, x_25); -if (lean_obj_tag(x_29) == 0) +lean_object* x_31; lean_object* x_32; +lean_dec(x_3); +x_31 = l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___lambda__2___closed__1; +x_32 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_32, 0, x_31); +lean_ctor_set(x_32, 1, x_8); +return x_32; +} +} +} +} +else { -lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_30 = lean_ctor_get(x_29, 0); -lean_inc(x_30); -x_31 = lean_ctor_get(x_29, 1); -lean_inc(x_31); -lean_dec(x_29); -x_32 = lean_apply_7(x_2, x_21, x_22, x_23, x_30, x_5, x_6, x_31); -if (lean_obj_tag(x_32) == 0) +switch (lean_obj_tag(x_3)) { +case 1: { uint8_t x_33; -x_33 = !lean_is_exclusive(x_32); +x_33 = !lean_is_exclusive(x_3); if (x_33 == 0) { -lean_object* x_34; lean_object* x_35; -x_34 = lean_ctor_get(x_32, 0); -x_35 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_35, 0, x_34); -lean_ctor_set(x_32, 0, x_35); -return x_32; +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_3, 0); +lean_dec(x_34); +x_35 = lean_ctor_get(x_12, 0); +lean_inc(x_35); +lean_dec(x_12); +lean_ctor_set(x_3, 0, x_35); +x_36 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_36, 0, x_3); +lean_ctor_set(x_36, 1, x_8); +return x_36; } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_36 = lean_ctor_get(x_32, 0); -x_37 = lean_ctor_get(x_32, 1); +lean_object* x_37; lean_object* x_38; lean_object* x_39; +lean_dec(x_3); +x_37 = lean_ctor_get(x_12, 0); lean_inc(x_37); -lean_inc(x_36); -lean_dec(x_32); +lean_dec(x_12); x_38 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_38, 0, x_36); +lean_ctor_set(x_38, 0, x_37); x_39 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_39, 0, x_38); -lean_ctor_set(x_39, 1, x_37); +lean_ctor_set(x_39, 1, x_8); return x_39; } } -else +case 3: { uint8_t x_40; -x_40 = !lean_is_exclusive(x_32); +x_40 = !lean_is_exclusive(x_12); if (x_40 == 0) { -return x_32; +lean_object* x_41; lean_object* x_42; uint8_t x_43; +x_41 = lean_ctor_get(x_12, 0); +x_42 = lean_ctor_get(x_12, 1); +lean_dec(x_42); +x_43 = !lean_is_exclusive(x_3); +if (x_43 == 0) +{ +lean_object* x_44; lean_object* x_45; +x_44 = lean_ctor_get(x_3, 0); +lean_ctor_set(x_12, 1, x_41); +lean_ctor_set(x_12, 0, x_44); +lean_ctor_set_tag(x_3, 1); +lean_ctor_set(x_3, 0, x_12); +x_45 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_45, 0, x_3); +lean_ctor_set(x_45, 1, x_8); +return x_45; } else { -lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_ctor_get(x_32, 0); -x_42 = lean_ctor_get(x_32, 1); -lean_inc(x_42); -lean_inc(x_41); -lean_dec(x_32); -x_43 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_43, 0, x_41); -lean_ctor_set(x_43, 1, x_42); -return x_43; -} +lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_46 = lean_ctor_get(x_3, 0); +lean_inc(x_46); +lean_dec(x_3); +lean_ctor_set(x_12, 1, x_41); +lean_ctor_set(x_12, 0, x_46); +x_47 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_47, 0, x_12); +x_48 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_48, 0, x_47); +lean_ctor_set(x_48, 1, x_8); +return x_48; } } else { -uint8_t x_44; -lean_dec(x_23); -lean_dec(x_22); -lean_dec(x_21); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_2); -x_44 = !lean_is_exclusive(x_29); -if (x_44 == 0) +lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_49 = lean_ctor_get(x_12, 0); +lean_inc(x_49); +lean_dec(x_12); +x_50 = lean_ctor_get(x_3, 0); +lean_inc(x_50); +if (lean_is_exclusive(x_3)) { + lean_ctor_release(x_3, 0); + x_51 = x_3; +} else { + lean_dec_ref(x_3); + x_51 = lean_box(0); +} +x_52 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_52, 0, x_50); +lean_ctor_set(x_52, 1, x_49); +if (lean_is_scalar(x_51)) { + x_53 = lean_alloc_ctor(1, 1, 0); +} else { + x_53 = x_51; + lean_ctor_set_tag(x_53, 1); +} +lean_ctor_set(x_53, 0, x_52); +x_54 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_54, 0, x_53); +lean_ctor_set(x_54, 1, x_8); +return x_54; +} +} +default: { -return x_29; +uint8_t x_55; +x_55 = !lean_is_exclusive(x_3); +if (x_55 == 0) +{ +lean_object* x_56; lean_object* x_57; lean_object* x_58; +x_56 = lean_ctor_get(x_3, 0); +lean_dec(x_56); +x_57 = lean_ctor_get(x_12, 0); +lean_inc(x_57); +lean_dec(x_12); +lean_ctor_set_tag(x_3, 1); +lean_ctor_set(x_3, 0, x_57); +x_58 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_58, 0, x_3); +lean_ctor_set(x_58, 1, x_8); +return x_58; } else { -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_29, 0); -x_46 = lean_ctor_get(x_29, 1); -lean_inc(x_46); -lean_inc(x_45); -lean_dec(x_29); -x_47 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_47, 0, x_45); -lean_ctor_set(x_47, 1, x_46); -return x_47; +lean_object* x_59; lean_object* x_60; lean_object* x_61; +lean_dec(x_3); +x_59 = lean_ctor_get(x_12, 0); +lean_inc(x_59); +lean_dec(x_12); +x_60 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_60, 0, x_59); +x_61 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_61, 0, x_60); +lean_ctor_set(x_61, 1, x_8); +return x_61; +} +} +} +} +} +} +static lean_object* _init_l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___lambda__1___boxed), 6, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_6 = lean_alloc_closure((void*)(l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___lambda__2___boxed), 8, 1); +lean_closure_set(x_6, 0, x_1); +x_7 = lean_box(0); +x_8 = l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___closed__1; +x_9 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__7(x_8, x_6, x_7, x_2, x_3, x_4, x_5); +return x_9; } } +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; +x_6 = l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6(x_1, x_2, x_3, x_4, x_5); +if (lean_obj_tag(x_6) == 0) +{ +lean_object* x_7; +x_7 = lean_ctor_get(x_6, 0); +lean_inc(x_7); +if (lean_obj_tag(x_7) == 0) +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) +{ +lean_object* x_9; lean_object* x_10; +x_9 = lean_ctor_get(x_6, 0); +lean_dec(x_9); +x_10 = lean_box(0); +lean_ctor_set(x_6, 0, x_10); +return x_6; } else { -uint8_t x_48; -lean_dec(x_23); -lean_dec(x_22); -lean_free_object(x_3); -lean_dec(x_21); +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_6, 1); +lean_inc(x_11); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_2); -lean_dec(x_1); -x_48 = !lean_is_exclusive(x_24); -if (x_48 == 0) +x_12 = lean_box(0); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_11); +return x_13; +} +} +else { -return x_24; +lean_object* x_14; +x_14 = lean_ctor_get(x_7, 0); +lean_inc(x_14); +lean_dec(x_7); +if (lean_obj_tag(x_14) == 0) +{ +uint8_t x_15; +x_15 = !lean_is_exclusive(x_6); +if (x_15 == 0) +{ +lean_object* x_16; lean_object* x_17; +x_16 = lean_ctor_get(x_6, 0); +lean_dec(x_16); +x_17 = lean_box(0); +lean_ctor_set(x_6, 0, x_17); +return x_6; } else { -lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_49 = lean_ctor_get(x_24, 0); -x_50 = lean_ctor_get(x_24, 1); -lean_inc(x_50); -lean_inc(x_49); -lean_dec(x_24); -x_51 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_51, 0, x_49); -lean_ctor_set(x_51, 1, x_50); -return x_51; -} +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_6, 1); +lean_inc(x_18); +lean_dec(x_6); +x_19 = lean_box(0); +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_19); +lean_ctor_set(x_20, 1, x_18); +return x_20; } } else { -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_52 = lean_ctor_get(x_3, 0); -lean_inc(x_52); -lean_dec(x_3); -x_53 = lean_ctor_get(x_4, 0); -lean_inc(x_53); -x_54 = lean_ctor_get(x_4, 1); -lean_inc(x_54); -lean_dec(x_4); -lean_inc(x_1); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_54); -lean_inc(x_53); -lean_inc(x_52); -x_55 = lean_apply_6(x_1, x_52, x_53, x_54, x_5, x_6, x_7); -if (lean_obj_tag(x_55) == 0) -{ -lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; -x_56 = lean_ctor_get(x_55, 1); -lean_inc(x_56); -lean_dec(x_55); -lean_inc(x_52); -x_57 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_57, 0, x_52); -x_58 = l_Lean_Elab_Info_updateContext_x3f(x_57, x_53); -x_59 = l_Lean_PersistentArray_toList___rarg(x_54); -x_60 = lean_box(0); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_2); -x_61 = l_List_mapM_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__9(x_1, x_2, x_58, x_59, x_60, x_5, x_6, x_56); -if (lean_obj_tag(x_61) == 0) +uint8_t x_21; +x_21 = !lean_is_exclusive(x_6); +if (x_21 == 0) { -lean_object* x_62; lean_object* x_63; lean_object* x_64; -x_62 = lean_ctor_get(x_61, 0); -lean_inc(x_62); -x_63 = lean_ctor_get(x_61, 1); -lean_inc(x_63); -lean_dec(x_61); -x_64 = lean_apply_7(x_2, x_52, x_53, x_54, x_62, x_5, x_6, x_63); -if (lean_obj_tag(x_64) == 0) +lean_object* x_22; uint8_t x_23; +x_22 = lean_ctor_get(x_6, 0); +lean_dec(x_22); +x_23 = !lean_is_exclusive(x_14); +if (x_23 == 0) { -lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_65 = lean_ctor_get(x_64, 0); -lean_inc(x_65); -x_66 = lean_ctor_get(x_64, 1); -lean_inc(x_66); -if (lean_is_exclusive(x_64)) { - lean_ctor_release(x_64, 0); - lean_ctor_release(x_64, 1); - x_67 = x_64; -} else { - lean_dec_ref(x_64); - x_67 = lean_box(0); -} -x_68 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_68, 0, x_65); -if (lean_is_scalar(x_67)) { - x_69 = lean_alloc_ctor(0, 2, 0); -} else { - x_69 = x_67; -} -lean_ctor_set(x_69, 0, x_68); -lean_ctor_set(x_69, 1, x_66); -return x_69; +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_14, 0); +x_25 = l_List_reverse___rarg(x_24); +lean_ctor_set(x_14, 0, x_25); +lean_ctor_set(x_6, 0, x_14); +return x_6; } else { -lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_70 = lean_ctor_get(x_64, 0); -lean_inc(x_70); -x_71 = lean_ctor_get(x_64, 1); -lean_inc(x_71); -if (lean_is_exclusive(x_64)) { - lean_ctor_release(x_64, 0); - lean_ctor_release(x_64, 1); - x_72 = x_64; -} else { - lean_dec_ref(x_64); - x_72 = lean_box(0); -} -if (lean_is_scalar(x_72)) { - x_73 = lean_alloc_ctor(1, 2, 0); -} else { - x_73 = x_72; -} -lean_ctor_set(x_73, 0, x_70); -lean_ctor_set(x_73, 1, x_71); -return x_73; +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_14, 0); +lean_inc(x_26); +lean_dec(x_14); +x_27 = l_List_reverse___rarg(x_26); +x_28 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_6, 0, x_28); +return x_6; } } else { -lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; -lean_dec(x_54); -lean_dec(x_53); -lean_dec(x_52); +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_29 = lean_ctor_get(x_6, 1); +lean_inc(x_29); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_2); -x_74 = lean_ctor_get(x_61, 0); -lean_inc(x_74); -x_75 = lean_ctor_get(x_61, 1); -lean_inc(x_75); -if (lean_is_exclusive(x_61)) { - lean_ctor_release(x_61, 0); - lean_ctor_release(x_61, 1); - x_76 = x_61; +x_30 = lean_ctor_get(x_14, 0); +lean_inc(x_30); +if (lean_is_exclusive(x_14)) { + lean_ctor_release(x_14, 0); + x_31 = x_14; } else { - lean_dec_ref(x_61); - x_76 = lean_box(0); + lean_dec_ref(x_14); + x_31 = lean_box(0); } -if (lean_is_scalar(x_76)) { - x_77 = lean_alloc_ctor(1, 2, 0); +x_32 = l_List_reverse___rarg(x_30); +if (lean_is_scalar(x_31)) { + x_33 = lean_alloc_ctor(1, 1, 0); } else { - x_77 = x_76; -} -lean_ctor_set(x_77, 0, x_74); -lean_ctor_set(x_77, 1, x_75); -return x_77; -} + x_33 = x_31; } -else -{ -lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; -lean_dec(x_54); -lean_dec(x_53); -lean_dec(x_52); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_2); -lean_dec(x_1); -x_78 = lean_ctor_get(x_55, 0); -lean_inc(x_78); -x_79 = lean_ctor_get(x_55, 1); -lean_inc(x_79); -if (lean_is_exclusive(x_55)) { - lean_ctor_release(x_55, 0); - lean_ctor_release(x_55, 1); - x_80 = x_55; -} else { - lean_dec_ref(x_55); - x_80 = lean_box(0); +lean_ctor_set(x_33, 0, x_32); +x_34 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_34, 0, x_33); +lean_ctor_set(x_34, 1, x_29); +return x_34; } -if (lean_is_scalar(x_80)) { - x_81 = lean_alloc_ctor(1, 2, 0); -} else { - x_81 = x_80; } -lean_ctor_set(x_81, 0, x_78); -lean_ctor_set(x_81, 1, x_79); -return x_81; } } +else +{ +uint8_t x_35; +x_35 = !lean_is_exclusive(x_6); +if (x_35 == 0) +{ +return x_6; } -default: +else { -lean_object* x_82; lean_object* x_83; +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_6, 0); +x_37 = lean_ctor_get(x_6, 1); +lean_inc(x_37); +lean_inc(x_36); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_82 = lean_box(0); -x_83 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_83, 0, x_82); -lean_ctor_set(x_83, 1, x_7); -return x_83; -} +x_38 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_38, 0, x_36); +lean_ctor_set(x_38, 1, x_37); +return x_38; } } } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6) { _start: { -lean_object* x_7; lean_object* x_8; -x_7 = lean_box(0); -x_8 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__7(x_1, x_2, x_7, x_3, x_4, x_5, x_6); -return x_8; -} -} -LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: +uint8_t x_7; +x_7 = lean_usize_dec_eq(x_5, x_6); +if (x_7 == 0) { -lean_object* x_7; lean_object* x_8; -x_7 = lean_box(0); -x_8 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_8, 0, x_7); -lean_ctor_set(x_8, 1, x_6); -return x_8; -} -} -static lean_object* _init_l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___lambda__2___closed__1() { -_start: +lean_object* x_8; lean_object* x_9; uint8_t x_10; +x_8 = lean_array_uget(x_4, x_5); +lean_inc(x_2); +lean_inc(x_3); +lean_inc(x_1); +x_9 = lean_apply_3(x_8, x_1, x_3, x_2); +x_10 = lean_unbox(x_9); +lean_dec(x_9); +if (x_10 == 0) { -lean_object* x_1; lean_object* x_2; -x_1 = lean_box(0); -x_2 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} +size_t x_11; size_t x_12; +x_11 = 1; +x_12 = lean_usize_add(x_5, x_11); +x_5 = x_12; +goto _start; } -LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_9 = lean_box(0); -x_10 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_340____closed__1; -x_11 = l_List_filterMapTR_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__1(x_5, x_10); -x_12 = l_List_filterMapTR_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__2(x_11, x_10); -if (lean_obj_tag(x_12) == 0) -{ -lean_object* x_13; uint8_t x_14; uint8_t x_15; -x_13 = lean_ctor_get(x_1, 0); -x_14 = 0; -x_15 = l_Lean_Elab_Info_contains(x_3, x_13, x_14); -if (x_15 == 0) +else { -lean_object* x_16; lean_object* x_17; +uint8_t x_14; lean_dec(x_3); -x_16 = lean_box(0); -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_16); -lean_ctor_set(x_17, 1, x_8); -return x_17; +lean_dec(x_2); +lean_dec(x_1); +x_14 = 1; +return x_14; +} } else { -lean_object* x_18; uint8_t x_19; uint8_t x_20; -x_18 = lean_ctor_get(x_1, 1); -x_19 = 1; -x_20 = l_Lean_Elab_Info_contains(x_3, x_18, x_19); -if (x_20 == 0) -{ -lean_object* x_21; lean_object* x_22; +uint8_t x_15; lean_dec(x_3); -x_21 = lean_box(0); -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_21); -lean_ctor_set(x_22, 1, x_8); -return x_22; +lean_dec(x_2); +lean_dec(x_1); +x_15 = 0; +return x_15; } -else +} +} +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__11(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6) { +_start: { -if (lean_obj_tag(x_3) == 3) +uint8_t x_7; +x_7 = lean_usize_dec_eq(x_5, x_6); +if (x_7 == 0) { -uint8_t x_23; -x_23 = !lean_is_exclusive(x_3); -if (x_23 == 0) +lean_object* x_8; lean_object* x_9; lean_object* x_10; uint64_t x_11; uint64_t x_12; uint64_t x_13; uint64_t x_14; uint64_t x_15; uint64_t x_16; uint64_t x_17; size_t x_18; size_t x_19; size_t x_20; size_t x_21; size_t x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; uint64_t x_27; uint64_t x_28; uint64_t x_29; uint64_t x_30; uint64_t x_31; size_t x_32; size_t x_33; size_t x_34; size_t x_35; lean_object* x_36; uint8_t x_37; +x_8 = lean_array_uget(x_4, x_5); +x_9 = lean_ctor_get(x_2, 1); +x_10 = lean_array_get_size(x_9); +x_11 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_8); +x_12 = 32; +x_13 = lean_uint64_shift_right(x_11, x_12); +x_14 = lean_uint64_xor(x_11, x_13); +x_15 = 16; +x_16 = lean_uint64_shift_right(x_14, x_15); +x_17 = lean_uint64_xor(x_14, x_16); +x_18 = lean_uint64_to_usize(x_17); +x_19 = lean_usize_of_nat(x_10); +lean_dec(x_10); +x_20 = 1; +x_21 = lean_usize_sub(x_19, x_20); +x_22 = lean_usize_land(x_18, x_21); +x_23 = lean_array_uget(x_9, x_22); +x_24 = l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__3(x_8, x_8, x_23); +lean_dec(x_23); +lean_dec(x_8); +x_25 = lean_ctor_get(x_3, 1); +x_26 = lean_array_get_size(x_25); +x_27 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_24); +x_28 = lean_uint64_shift_right(x_27, x_12); +x_29 = lean_uint64_xor(x_27, x_28); +x_30 = lean_uint64_shift_right(x_29, x_15); +x_31 = lean_uint64_xor(x_29, x_30); +x_32 = lean_uint64_to_usize(x_31); +x_33 = lean_usize_of_nat(x_26); +lean_dec(x_26); +x_34 = lean_usize_sub(x_33, x_20); +x_35 = lean_usize_land(x_32, x_34); +x_36 = lean_array_uget(x_25, x_35); +x_37 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_24, x_36); +lean_dec(x_36); +lean_dec(x_24); +if (x_37 == 0) { -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_3, 0); -x_25 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_25, 0, x_24); -lean_ctor_set(x_25, 1, x_9); -lean_ctor_set_tag(x_3, 1); -lean_ctor_set(x_3, 0, x_25); -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_3); -lean_ctor_set(x_26, 1, x_8); -return x_26; +size_t x_38; +x_38 = lean_usize_add(x_5, x_20); +x_5 = x_38; +goto _start; } else { -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_27 = lean_ctor_get(x_3, 0); -lean_inc(x_27); -lean_dec(x_3); -x_28 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_28, 0, x_27); -lean_ctor_set(x_28, 1, x_9); -x_29 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_29, 0, x_28); -x_30 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_30, 0, x_29); -lean_ctor_set(x_30, 1, x_8); -return x_30; +uint8_t x_40; +x_40 = 1; +return x_40; } } else { -lean_object* x_31; lean_object* x_32; -lean_dec(x_3); -x_31 = l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___lambda__2___closed__1; -x_32 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_32, 0, x_31); -lean_ctor_set(x_32, 1, x_8); -return x_32; -} +uint8_t x_41; +x_41 = 0; +return x_41; } } } -else -{ -switch (lean_obj_tag(x_3)) { -case 1: +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__12(lean_object* x_1, lean_object* x_2) { +_start: { -uint8_t x_33; -x_33 = !lean_is_exclusive(x_3); -if (x_33 == 0) +if (lean_obj_tag(x_2) == 0) { -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_3, 0); -lean_dec(x_34); -x_35 = lean_ctor_get(x_12, 0); -lean_inc(x_35); -lean_dec(x_12); -lean_ctor_set(x_3, 0, x_35); -x_36 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_36, 0, x_3); -lean_ctor_set(x_36, 1, x_8); -return x_36; +return x_1; } else { -lean_object* x_37; lean_object* x_38; lean_object* x_39; -lean_dec(x_3); -x_37 = lean_ctor_get(x_12, 0); -lean_inc(x_37); -lean_dec(x_12); -x_38 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_38, 0, x_37); -x_39 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_39, 0, x_38); -lean_ctor_set(x_39, 1, x_8); -return x_39; +lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_3 = lean_ctor_get(x_2, 0); +lean_inc(x_3); +x_4 = lean_ctor_get(x_2, 2); +lean_inc(x_4); +lean_dec(x_2); +x_5 = lean_array_push(x_1, x_3); +x_1 = x_5; +x_2 = x_4; +goto _start; } } -case 3: -{ -uint8_t x_40; -x_40 = !lean_is_exclusive(x_12); -if (x_40 == 0) +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__13(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: { -lean_object* x_41; lean_object* x_42; uint8_t x_43; -x_41 = lean_ctor_get(x_12, 0); -x_42 = lean_ctor_get(x_12, 1); -lean_dec(x_42); -x_43 = !lean_is_exclusive(x_3); -if (x_43 == 0) +if (lean_obj_tag(x_3) == 0) { -lean_object* x_44; lean_object* x_45; -x_44 = lean_ctor_get(x_3, 0); -lean_ctor_set(x_12, 1, x_41); -lean_ctor_set(x_12, 0, x_44); -lean_ctor_set_tag(x_3, 1); -lean_ctor_set(x_3, 0, x_12); -x_45 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_45, 0, x_3); -lean_ctor_set(x_45, 1, x_8); -return x_45; +lean_object* x_4; +lean_dec(x_2); +lean_dec(x_1); +x_4 = lean_box(0); +return x_4; } else { -lean_object* x_46; lean_object* x_47; lean_object* x_48; -x_46 = lean_ctor_get(x_3, 0); -lean_inc(x_46); -lean_dec(x_3); -lean_ctor_set(x_12, 1, x_41); -lean_ctor_set(x_12, 0, x_46); -x_47 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_47, 0, x_12); -x_48 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_48, 0, x_47); -lean_ctor_set(x_48, 1, x_8); -return x_48; -} +uint8_t x_5; +x_5 = !lean_is_exclusive(x_3); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; +x_6 = lean_ctor_get(x_3, 0); +x_7 = lean_ctor_get(x_3, 1); +x_8 = lean_ctor_get(x_3, 2); +x_9 = lean_name_eq(x_6, x_1); +if (x_9 == 0) +{ +lean_object* x_10; +x_10 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__13(x_1, x_2, x_8); +lean_ctor_set(x_3, 2, x_10); +return x_3; } else { -lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; -x_49 = lean_ctor_get(x_12, 0); -lean_inc(x_49); -lean_dec(x_12); -x_50 = lean_ctor_get(x_3, 0); -lean_inc(x_50); -if (lean_is_exclusive(x_3)) { - lean_ctor_release(x_3, 0); - x_51 = x_3; -} else { - lean_dec_ref(x_3); - x_51 = lean_box(0); -} -x_52 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_52, 0, x_50); -lean_ctor_set(x_52, 1, x_49); -if (lean_is_scalar(x_51)) { - x_53 = lean_alloc_ctor(1, 1, 0); -} else { - x_53 = x_51; - lean_ctor_set_tag(x_53, 1); -} -lean_ctor_set(x_53, 0, x_52); -x_54 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_54, 0, x_53); -lean_ctor_set(x_54, 1, x_8); -return x_54; +lean_dec(x_7); +lean_dec(x_6); +lean_ctor_set(x_3, 1, x_2); +lean_ctor_set(x_3, 0, x_1); +return x_3; } } -default: +else { -uint8_t x_55; -x_55 = !lean_is_exclusive(x_3); -if (x_55 == 0) +lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_11 = lean_ctor_get(x_3, 0); +x_12 = lean_ctor_get(x_3, 1); +x_13 = lean_ctor_get(x_3, 2); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_dec(x_3); +x_14 = lean_name_eq(x_11, x_1); +if (x_14 == 0) { -lean_object* x_56; lean_object* x_57; lean_object* x_58; -x_56 = lean_ctor_get(x_3, 0); -lean_dec(x_56); -x_57 = lean_ctor_get(x_12, 0); -lean_inc(x_57); -lean_dec(x_12); -lean_ctor_set_tag(x_3, 1); -lean_ctor_set(x_3, 0, x_57); -x_58 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_58, 0, x_3); -lean_ctor_set(x_58, 1, x_8); -return x_58; +lean_object* x_15; lean_object* x_16; +x_15 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__13(x_1, x_2, x_13); +x_16 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_16, 0, x_11); +lean_ctor_set(x_16, 1, x_12); +lean_ctor_set(x_16, 2, x_15); +return x_16; } else { -lean_object* x_59; lean_object* x_60; lean_object* x_61; -lean_dec(x_3); -x_59 = lean_ctor_get(x_12, 0); -lean_inc(x_59); +lean_object* x_17; lean_dec(x_12); -x_60 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_60, 0, x_59); -x_61 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_61, 0, x_60); -lean_ctor_set(x_61, 1, x_8); -return x_61; -} +lean_dec(x_11); +x_17 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_17, 0, x_1); +lean_ctor_set(x_17, 1, x_2); +lean_ctor_set(x_17, 2, x_13); +return x_17; } } } } } -static lean_object* _init_l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___closed__1() { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__14(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___lambda__1___boxed), 6, 0); -return x_1; +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_3, x_2); +if (x_5 == 0) +{ +return x_4; } +else +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; size_t x_9; size_t x_10; lean_object* x_11; lean_object* x_12; uint64_t x_13; uint64_t x_14; uint64_t x_15; uint64_t x_16; uint64_t x_17; uint64_t x_18; uint64_t x_19; size_t x_20; size_t x_21; size_t x_22; size_t x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_6 = lean_array_uget(x_4, x_3); +x_7 = lean_unsigned_to_nat(0u); +x_8 = lean_array_uset(x_4, x_3, x_7); +x_9 = 1; +x_10 = lean_usize_add(x_3, x_9); +x_11 = lean_ctor_get(x_1, 1); +x_12 = lean_array_get_size(x_11); +x_13 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_6); +x_14 = 32; +x_15 = lean_uint64_shift_right(x_13, x_14); +x_16 = lean_uint64_xor(x_13, x_15); +x_17 = 16; +x_18 = lean_uint64_shift_right(x_16, x_17); +x_19 = lean_uint64_xor(x_16, x_18); +x_20 = lean_uint64_to_usize(x_19); +x_21 = lean_usize_of_nat(x_12); +lean_dec(x_12); +x_22 = lean_usize_sub(x_21, x_9); +x_23 = lean_usize_land(x_20, x_22); +x_24 = lean_array_uget(x_11, x_23); +x_25 = l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__3(x_6, x_6, x_24); +lean_dec(x_24); +lean_dec(x_6); +x_26 = lean_array_uset(x_8, x_3, x_25); +x_3 = x_10; +x_4 = x_26; +goto _start; } -LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_6 = lean_alloc_closure((void*)(l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___lambda__2___boxed), 8, 1); -lean_closure_set(x_6, 0, x_1); -x_7 = l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___closed__1; -x_8 = l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6(x_7, x_6, x_2, x_3, x_4, x_5); -return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6) { _start: { -lean_object* x_6; -x_6 = l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5(x_1, x_2, x_3, x_4, x_5); -if (lean_obj_tag(x_6) == 0) -{ -lean_object* x_7; -x_7 = lean_ctor_get(x_6, 0); -lean_inc(x_7); -if (lean_obj_tag(x_7) == 0) -{ -uint8_t x_8; -x_8 = !lean_is_exclusive(x_6); -if (x_8 == 0) +uint8_t x_7; +x_7 = lean_usize_dec_lt(x_5, x_4); +if (x_7 == 0) { -lean_object* x_9; lean_object* x_10; -x_9 = lean_ctor_get(x_6, 0); -lean_dec(x_9); -x_10 = lean_box(0); -lean_ctor_set(x_6, 0, x_10); +lean_dec(x_1); return x_6; } else { -lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_11 = lean_ctor_get(x_6, 1); -lean_inc(x_11); -lean_dec(x_6); -x_12 = lean_box(0); -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_12); -lean_ctor_set(x_13, 1, x_11); -return x_13; -} -} -else +lean_object* x_8; uint8_t x_9; +x_8 = lean_array_uget(x_3, x_5); +x_9 = !lean_is_exclusive(x_6); +if (x_9 == 0) { -lean_object* x_14; -x_14 = lean_ctor_get(x_7, 0); -lean_inc(x_14); -lean_dec(x_7); -if (lean_obj_tag(x_14) == 0) +lean_object* x_10; lean_object* x_11; lean_object* x_12; uint64_t x_13; uint64_t x_14; uint64_t x_15; uint64_t x_16; uint64_t x_17; uint64_t x_18; uint64_t x_19; size_t x_20; size_t x_21; size_t x_22; size_t x_23; size_t x_24; lean_object* x_25; uint8_t x_26; +x_10 = lean_ctor_get(x_6, 0); +x_11 = lean_ctor_get(x_6, 1); +x_12 = lean_array_get_size(x_11); +x_13 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_8); +x_14 = 32; +x_15 = lean_uint64_shift_right(x_13, x_14); +x_16 = lean_uint64_xor(x_13, x_15); +x_17 = 16; +x_18 = lean_uint64_shift_right(x_16, x_17); +x_19 = lean_uint64_xor(x_16, x_18); +x_20 = lean_uint64_to_usize(x_19); +x_21 = lean_usize_of_nat(x_12); +lean_dec(x_12); +x_22 = 1; +x_23 = lean_usize_sub(x_21, x_22); +x_24 = lean_usize_land(x_20, x_23); +x_25 = lean_array_uget(x_11, x_24); +x_26 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_8, x_25); +if (x_26 == 0) { -uint8_t x_15; -x_15 = !lean_is_exclusive(x_6); -if (x_15 == 0) +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; +x_27 = lean_unsigned_to_nat(1u); +x_28 = lean_nat_add(x_10, x_27); +lean_dec(x_10); +x_29 = lean_box(0); +x_30 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_30, 0, x_8); +lean_ctor_set(x_30, 1, x_29); +lean_ctor_set(x_30, 2, x_25); +x_31 = lean_array_uset(x_11, x_24, x_30); +x_32 = lean_unsigned_to_nat(4u); +x_33 = lean_nat_mul(x_28, x_32); +x_34 = lean_unsigned_to_nat(3u); +x_35 = lean_nat_div(x_33, x_34); +lean_dec(x_33); +x_36 = lean_array_get_size(x_31); +x_37 = lean_nat_dec_le(x_35, x_36); +lean_dec(x_36); +lean_dec(x_35); +if (x_37 == 0) { -lean_object* x_16; lean_object* x_17; -x_16 = lean_ctor_get(x_6, 0); -lean_dec(x_16); -x_17 = lean_box(0); -lean_ctor_set(x_6, 0, x_17); -return x_6; +lean_object* x_38; size_t x_39; +x_38 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_31); +lean_ctor_set(x_6, 1, x_38); +lean_ctor_set(x_6, 0, x_28); +x_39 = lean_usize_add(x_5, x_22); +x_5 = x_39; +goto _start; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_6, 1); -lean_inc(x_18); -lean_dec(x_6); -x_19 = lean_box(0); -x_20 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_20, 0, x_19); -lean_ctor_set(x_20, 1, x_18); -return x_20; +size_t x_41; +lean_ctor_set(x_6, 1, x_31); +lean_ctor_set(x_6, 0, x_28); +x_41 = lean_usize_add(x_5, x_22); +x_5 = x_41; +goto _start; } } else { -uint8_t x_21; -x_21 = !lean_is_exclusive(x_6); -if (x_21 == 0) +lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; size_t x_47; +lean_inc(x_1); +x_43 = lean_array_uset(x_11, x_24, x_1); +x_44 = lean_box(0); +x_45 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__13(x_8, x_44, x_25); +x_46 = lean_array_uset(x_43, x_24, x_45); +lean_ctor_set(x_6, 1, x_46); +x_47 = lean_usize_add(x_5, x_22); +x_5 = x_47; +goto _start; +} +} +else { -lean_object* x_22; uint8_t x_23; -x_22 = lean_ctor_get(x_6, 0); -lean_dec(x_22); -x_23 = !lean_is_exclusive(x_14); -if (x_23 == 0) +lean_object* x_49; lean_object* x_50; lean_object* x_51; uint64_t x_52; uint64_t x_53; uint64_t x_54; uint64_t x_55; uint64_t x_56; uint64_t x_57; uint64_t x_58; size_t x_59; size_t x_60; size_t x_61; size_t x_62; size_t x_63; lean_object* x_64; uint8_t x_65; +x_49 = lean_ctor_get(x_6, 0); +x_50 = lean_ctor_get(x_6, 1); +lean_inc(x_50); +lean_inc(x_49); +lean_dec(x_6); +x_51 = lean_array_get_size(x_50); +x_52 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_8); +x_53 = 32; +x_54 = lean_uint64_shift_right(x_52, x_53); +x_55 = lean_uint64_xor(x_52, x_54); +x_56 = 16; +x_57 = lean_uint64_shift_right(x_55, x_56); +x_58 = lean_uint64_xor(x_55, x_57); +x_59 = lean_uint64_to_usize(x_58); +x_60 = lean_usize_of_nat(x_51); +lean_dec(x_51); +x_61 = 1; +x_62 = lean_usize_sub(x_60, x_61); +x_63 = lean_usize_land(x_59, x_62); +x_64 = lean_array_uget(x_50, x_63); +x_65 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_8, x_64); +if (x_65 == 0) +{ +lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; uint8_t x_76; +x_66 = lean_unsigned_to_nat(1u); +x_67 = lean_nat_add(x_49, x_66); +lean_dec(x_49); +x_68 = lean_box(0); +x_69 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_69, 0, x_8); +lean_ctor_set(x_69, 1, x_68); +lean_ctor_set(x_69, 2, x_64); +x_70 = lean_array_uset(x_50, x_63, x_69); +x_71 = lean_unsigned_to_nat(4u); +x_72 = lean_nat_mul(x_67, x_71); +x_73 = lean_unsigned_to_nat(3u); +x_74 = lean_nat_div(x_72, x_73); +lean_dec(x_72); +x_75 = lean_array_get_size(x_70); +x_76 = lean_nat_dec_le(x_74, x_75); +lean_dec(x_75); +lean_dec(x_74); +if (x_76 == 0) { -lean_object* x_24; lean_object* x_25; -x_24 = lean_ctor_get(x_14, 0); -x_25 = l_List_reverse___rarg(x_24); -lean_ctor_set(x_14, 0, x_25); -lean_ctor_set(x_6, 0, x_14); -return x_6; +lean_object* x_77; lean_object* x_78; size_t x_79; +x_77 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_70); +x_78 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_78, 0, x_67); +lean_ctor_set(x_78, 1, x_77); +x_79 = lean_usize_add(x_5, x_61); +x_5 = x_79; +x_6 = x_78; +goto _start; } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_14, 0); -lean_inc(x_26); -lean_dec(x_14); -x_27 = l_List_reverse___rarg(x_26); -x_28 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_28, 0, x_27); -lean_ctor_set(x_6, 0, x_28); -return x_6; +lean_object* x_81; size_t x_82; +x_81 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_81, 0, x_67); +lean_ctor_set(x_81, 1, x_70); +x_82 = lean_usize_add(x_5, x_61); +x_5 = x_82; +x_6 = x_81; +goto _start; } } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_29 = lean_ctor_get(x_6, 1); -lean_inc(x_29); -lean_dec(x_6); -x_30 = lean_ctor_get(x_14, 0); -lean_inc(x_30); -if (lean_is_exclusive(x_14)) { - lean_ctor_release(x_14, 0); - x_31 = x_14; -} else { - lean_dec_ref(x_14); - x_31 = lean_box(0); -} -x_32 = l_List_reverse___rarg(x_30); -if (lean_is_scalar(x_31)) { - x_33 = lean_alloc_ctor(1, 1, 0); -} else { - x_33 = x_31; +lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; size_t x_89; +lean_inc(x_1); +x_84 = lean_array_uset(x_50, x_63, x_1); +x_85 = lean_box(0); +x_86 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__13(x_8, x_85, x_64); +x_87 = lean_array_uset(x_84, x_63, x_86); +x_88 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_88, 0, x_49); +lean_ctor_set(x_88, 1, x_87); +x_89 = lean_usize_add(x_5, x_61); +x_5 = x_89; +x_6 = x_88; +goto _start; } -lean_ctor_set(x_33, 0, x_32); -x_34 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_34, 0, x_33); -lean_ctor_set(x_34, 1, x_29); -return x_34; } } } } -else +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +_start: { -uint8_t x_35; -x_35 = !lean_is_exclusive(x_6); -if (x_35 == 0) +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_3, x_2); +if (x_5 == 0) { -return x_6; +return x_4; } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_6, 0); -x_37 = lean_ctor_get(x_6, 1); -lean_inc(x_37); -lean_inc(x_36); +lean_object* x_6; lean_object* x_7; lean_object* x_8; size_t x_9; size_t x_10; lean_object* x_11; lean_object* x_12; uint64_t x_13; uint64_t x_14; uint64_t x_15; uint64_t x_16; uint64_t x_17; uint64_t x_18; uint64_t x_19; size_t x_20; size_t x_21; size_t x_22; size_t x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_6 = lean_array_uget(x_4, x_3); +x_7 = lean_unsigned_to_nat(0u); +x_8 = lean_array_uset(x_4, x_3, x_7); +x_9 = 1; +x_10 = lean_usize_add(x_3, x_9); +x_11 = lean_ctor_get(x_1, 1); +x_12 = lean_array_get_size(x_11); +x_13 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_6); +x_14 = 32; +x_15 = lean_uint64_shift_right(x_13, x_14); +x_16 = lean_uint64_xor(x_13, x_15); +x_17 = 16; +x_18 = lean_uint64_shift_right(x_16, x_17); +x_19 = lean_uint64_xor(x_16, x_18); +x_20 = lean_uint64_to_usize(x_19); +x_21 = lean_usize_of_nat(x_12); +lean_dec(x_12); +x_22 = lean_usize_sub(x_21, x_9); +x_23 = lean_usize_land(x_20, x_22); +x_24 = lean_array_uget(x_11, x_23); +x_25 = l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__3(x_6, x_6, x_24); +lean_dec(x_24); lean_dec(x_6); -x_38 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -return x_38; -} +x_26 = lean_array_uset(x_8, x_3, x_25); +x_3 = x_10; +x_4 = x_26; +goto _start; } } } -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__17(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6) { _start: { uint8_t x_7; -x_7 = lean_usize_dec_eq(x_5, x_6); +x_7 = lean_usize_dec_lt(x_5, x_4); if (x_7 == 0) { -lean_object* x_8; lean_object* x_9; uint8_t x_10; -x_8 = lean_array_uget(x_4, x_5); -lean_inc(x_2); -lean_inc(x_3); -lean_inc(x_1); -x_9 = lean_apply_3(x_8, x_1, x_3, x_2); -x_10 = lean_unbox(x_9); -lean_dec(x_9); -if (x_10 == 0) +lean_dec(x_1); +return x_6; +} +else +{ +lean_object* x_8; uint8_t x_9; +x_8 = lean_array_uget(x_3, x_5); +x_9 = !lean_is_exclusive(x_6); +if (x_9 == 0) +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; uint64_t x_13; uint64_t x_14; uint64_t x_15; uint64_t x_16; uint64_t x_17; uint64_t x_18; uint64_t x_19; size_t x_20; size_t x_21; size_t x_22; size_t x_23; size_t x_24; lean_object* x_25; uint8_t x_26; +x_10 = lean_ctor_get(x_6, 0); +x_11 = lean_ctor_get(x_6, 1); +x_12 = lean_array_get_size(x_11); +x_13 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_8); +x_14 = 32; +x_15 = lean_uint64_shift_right(x_13, x_14); +x_16 = lean_uint64_xor(x_13, x_15); +x_17 = 16; +x_18 = lean_uint64_shift_right(x_16, x_17); +x_19 = lean_uint64_xor(x_16, x_18); +x_20 = lean_uint64_to_usize(x_19); +x_21 = lean_usize_of_nat(x_12); +lean_dec(x_12); +x_22 = 1; +x_23 = lean_usize_sub(x_21, x_22); +x_24 = lean_usize_land(x_20, x_23); +x_25 = lean_array_uget(x_11, x_24); +x_26 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_8, x_25); +if (x_26 == 0) +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; +x_27 = lean_unsigned_to_nat(1u); +x_28 = lean_nat_add(x_10, x_27); +lean_dec(x_10); +x_29 = lean_box(0); +x_30 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_30, 0, x_8); +lean_ctor_set(x_30, 1, x_29); +lean_ctor_set(x_30, 2, x_25); +x_31 = lean_array_uset(x_11, x_24, x_30); +x_32 = lean_unsigned_to_nat(4u); +x_33 = lean_nat_mul(x_28, x_32); +x_34 = lean_unsigned_to_nat(3u); +x_35 = lean_nat_div(x_33, x_34); +lean_dec(x_33); +x_36 = lean_array_get_size(x_31); +x_37 = lean_nat_dec_le(x_35, x_36); +lean_dec(x_36); +lean_dec(x_35); +if (x_37 == 0) { -size_t x_11; size_t x_12; -x_11 = 1; -x_12 = lean_usize_add(x_5, x_11); -x_5 = x_12; +lean_object* x_38; size_t x_39; +x_38 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_31); +lean_ctor_set(x_6, 1, x_38); +lean_ctor_set(x_6, 0, x_28); +x_39 = lean_usize_add(x_5, x_22); +x_5 = x_39; goto _start; } else { -uint8_t x_14; -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_14 = 1; -return x_14; +size_t x_41; +lean_ctor_set(x_6, 1, x_31); +lean_ctor_set(x_6, 0, x_28); +x_41 = lean_usize_add(x_5, x_22); +x_5 = x_41; +goto _start; } } else { -uint8_t x_15; -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_15 = 0; -return x_15; -} +lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; size_t x_47; +lean_inc(x_1); +x_43 = lean_array_uset(x_11, x_24, x_1); +x_44 = lean_box(0); +x_45 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__13(x_8, x_44, x_25); +x_46 = lean_array_uset(x_43, x_24, x_45); +lean_ctor_set(x_6, 1, x_46); +x_47 = lean_usize_add(x_5, x_22); +x_5 = x_47; +goto _start; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__11(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: +else { -if (lean_obj_tag(x_3) == 0) +lean_object* x_49; lean_object* x_50; lean_object* x_51; uint64_t x_52; uint64_t x_53; uint64_t x_54; uint64_t x_55; uint64_t x_56; uint64_t x_57; uint64_t x_58; size_t x_59; size_t x_60; size_t x_61; size_t x_62; size_t x_63; lean_object* x_64; uint8_t x_65; +x_49 = lean_ctor_get(x_6, 0); +x_50 = lean_ctor_get(x_6, 1); +lean_inc(x_50); +lean_inc(x_49); +lean_dec(x_6); +x_51 = lean_array_get_size(x_50); +x_52 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_8); +x_53 = 32; +x_54 = lean_uint64_shift_right(x_52, x_53); +x_55 = lean_uint64_xor(x_52, x_54); +x_56 = 16; +x_57 = lean_uint64_shift_right(x_55, x_56); +x_58 = lean_uint64_xor(x_55, x_57); +x_59 = lean_uint64_to_usize(x_58); +x_60 = lean_usize_of_nat(x_51); +lean_dec(x_51); +x_61 = 1; +x_62 = lean_usize_sub(x_60, x_61); +x_63 = lean_usize_land(x_59, x_62); +x_64 = lean_array_uget(x_50, x_63); +x_65 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_8, x_64); +if (x_65 == 0) +{ +lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; uint8_t x_76; +x_66 = lean_unsigned_to_nat(1u); +x_67 = lean_nat_add(x_49, x_66); +lean_dec(x_49); +x_68 = lean_box(0); +x_69 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_69, 0, x_8); +lean_ctor_set(x_69, 1, x_68); +lean_ctor_set(x_69, 2, x_64); +x_70 = lean_array_uset(x_50, x_63, x_69); +x_71 = lean_unsigned_to_nat(4u); +x_72 = lean_nat_mul(x_67, x_71); +x_73 = lean_unsigned_to_nat(3u); +x_74 = lean_nat_div(x_72, x_73); +lean_dec(x_72); +x_75 = lean_array_get_size(x_70); +x_76 = lean_nat_dec_le(x_74, x_75); +lean_dec(x_75); +lean_dec(x_74); +if (x_76 == 0) { -lean_inc(x_2); -return x_2; +lean_object* x_77; lean_object* x_78; size_t x_79; +x_77 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_70); +x_78 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_78, 0, x_67); +lean_ctor_set(x_78, 1, x_77); +x_79 = lean_usize_add(x_5, x_61); +x_5 = x_79; +x_6 = x_78; +goto _start; } else { -lean_object* x_4; lean_object* x_5; lean_object* x_6; uint8_t x_7; -x_4 = lean_ctor_get(x_3, 0); -x_5 = lean_ctor_get(x_3, 1); -x_6 = lean_ctor_get(x_3, 2); -x_7 = lean_name_eq(x_4, x_1); -if (x_7 == 0) -{ -x_3 = x_6; +lean_object* x_81; size_t x_82; +x_81 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_81, 0, x_67); +lean_ctor_set(x_81, 1, x_70); +x_82 = lean_usize_add(x_5, x_61); +x_5 = x_82; +x_6 = x_81; goto _start; } +} else { -lean_inc(x_5); -return x_5; +lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; size_t x_89; +lean_inc(x_1); +x_84 = lean_array_uset(x_50, x_63, x_1); +x_85 = lean_box(0); +x_86 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__13(x_8, x_85, x_64); +x_87 = lean_array_uset(x_84, x_63, x_86); +x_88 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_88, 0, x_49); +lean_ctor_set(x_88, 1, x_87); +x_89 = lean_usize_add(x_5, x_61); +x_5 = x_89; +x_6 = x_88; +goto _start; } } } } -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__12(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6) { +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__18(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { -uint8_t x_7; -x_7 = lean_usize_dec_eq(x_5, x_6); -if (x_7 == 0) -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; uint64_t x_11; uint64_t x_12; uint64_t x_13; uint64_t x_14; uint64_t x_15; uint64_t x_16; uint64_t x_17; size_t x_18; size_t x_19; size_t x_20; size_t x_21; size_t x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; uint64_t x_27; uint64_t x_28; uint64_t x_29; uint64_t x_30; uint64_t x_31; size_t x_32; size_t x_33; size_t x_34; size_t x_35; lean_object* x_36; uint8_t x_37; -x_8 = lean_array_uget(x_4, x_5); -x_9 = lean_ctor_get(x_2, 1); -x_10 = lean_array_get_size(x_9); -x_11 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_8); -x_12 = 32; -x_13 = lean_uint64_shift_right(x_11, x_12); -x_14 = lean_uint64_xor(x_11, x_13); -x_15 = 16; -x_16 = lean_uint64_shift_right(x_14, x_15); -x_17 = lean_uint64_xor(x_14, x_16); -x_18 = lean_uint64_to_usize(x_17); -x_19 = lean_usize_of_nat(x_10); -lean_dec(x_10); -x_20 = 1; -x_21 = lean_usize_sub(x_19, x_20); -x_22 = lean_usize_land(x_18, x_21); -x_23 = lean_array_uget(x_9, x_22); -x_24 = l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__11(x_8, x_8, x_23); -lean_dec(x_23); -lean_dec(x_8); -x_25 = lean_ctor_get(x_3, 1); -x_26 = lean_array_get_size(x_25); -x_27 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_24); -x_28 = lean_uint64_shift_right(x_27, x_12); -x_29 = lean_uint64_xor(x_27, x_28); -x_30 = lean_uint64_shift_right(x_29, x_15); -x_31 = lean_uint64_xor(x_29, x_30); -x_32 = lean_uint64_to_usize(x_31); -x_33 = lean_usize_of_nat(x_26); -lean_dec(x_26); -x_34 = lean_usize_sub(x_33, x_20); -x_35 = lean_usize_land(x_32, x_34); -x_36 = lean_array_uget(x_25, x_35); -x_37 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_24, x_36); -lean_dec(x_36); -lean_dec(x_24); -if (x_37 == 0) +uint8_t x_5; +x_5 = lean_usize_dec_eq(x_2, x_3); +if (x_5 == 0) { -size_t x_38; -x_38 = lean_usize_add(x_5, x_20); -x_5 = x_38; +lean_object* x_6; lean_object* x_7; size_t x_8; size_t x_9; +x_6 = lean_array_uget(x_1, x_2); +x_7 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__12(x_4, x_6); +x_8 = 1; +x_9 = lean_usize_add(x_2, x_8); +x_2 = x_9; +x_4 = x_7; goto _start; } else { -uint8_t x_40; -x_40 = 1; -return x_40; -} -} -else -{ -uint8_t x_41; -x_41 = 0; -return x_41; +return x_4; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__13(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { -if (lean_obj_tag(x_4) == 0) -{ -return x_3; -} -else -{ uint8_t x_5; -x_5 = !lean_is_exclusive(x_4); +x_5 = lean_usize_dec_lt(x_3, x_2); if (x_5 == 0) { -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint64_t x_11; uint64_t x_12; uint64_t x_13; uint64_t x_14; uint64_t x_15; uint64_t x_16; uint64_t x_17; size_t x_18; size_t x_19; size_t x_20; size_t x_21; size_t x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; -x_6 = lean_ctor_get(x_4, 0); -x_7 = lean_ctor_get(x_4, 2); -x_8 = lean_ctor_get(x_4, 1); -lean_dec(x_8); -x_9 = lean_ctor_get(x_2, 1); -x_10 = lean_array_get_size(x_9); -x_11 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_6); -x_12 = 32; -x_13 = lean_uint64_shift_right(x_11, x_12); -x_14 = lean_uint64_xor(x_11, x_13); -x_15 = 16; -x_16 = lean_uint64_shift_right(x_14, x_15); -x_17 = lean_uint64_xor(x_14, x_16); -x_18 = lean_uint64_to_usize(x_17); -x_19 = lean_usize_of_nat(x_10); -lean_dec(x_10); -x_20 = 1; -x_21 = lean_usize_sub(x_19, x_20); -x_22 = lean_usize_land(x_18, x_21); -x_23 = lean_array_uget(x_9, x_22); -x_24 = l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__11(x_6, x_6, x_23); -lean_dec(x_23); -lean_dec(x_6); -x_25 = !lean_is_exclusive(x_3); -if (x_25 == 0) -{ -lean_object* x_26; lean_object* x_27; lean_object* x_28; uint64_t x_29; uint64_t x_30; uint64_t x_31; uint64_t x_32; uint64_t x_33; size_t x_34; size_t x_35; size_t x_36; size_t x_37; lean_object* x_38; uint8_t x_39; -x_26 = lean_ctor_get(x_3, 0); -x_27 = lean_ctor_get(x_3, 1); -x_28 = lean_array_get_size(x_27); -x_29 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_24); -x_30 = lean_uint64_shift_right(x_29, x_12); -x_31 = lean_uint64_xor(x_29, x_30); -x_32 = lean_uint64_shift_right(x_31, x_15); -x_33 = lean_uint64_xor(x_31, x_32); -x_34 = lean_uint64_to_usize(x_33); -x_35 = lean_usize_of_nat(x_28); -lean_dec(x_28); -x_36 = lean_usize_sub(x_35, x_20); -x_37 = lean_usize_land(x_34, x_36); -x_38 = lean_array_uget(x_27, x_37); -x_39 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_24, x_38); -if (x_39 == 0) -{ -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; -x_40 = lean_unsigned_to_nat(1u); -x_41 = lean_nat_add(x_26, x_40); -lean_dec(x_26); -x_42 = lean_box(0); -lean_ctor_set(x_4, 2, x_38); -lean_ctor_set(x_4, 1, x_42); -lean_ctor_set(x_4, 0, x_24); -x_43 = lean_array_uset(x_27, x_37, x_4); -x_44 = lean_unsigned_to_nat(4u); -x_45 = lean_nat_mul(x_41, x_44); -x_46 = lean_unsigned_to_nat(3u); -x_47 = lean_nat_div(x_45, x_46); -lean_dec(x_45); -x_48 = lean_array_get_size(x_43); -x_49 = lean_nat_dec_le(x_47, x_48); -lean_dec(x_48); -lean_dec(x_47); -if (x_49 == 0) -{ -lean_object* x_50; -x_50 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_43); -lean_ctor_set(x_3, 1, x_50); -lean_ctor_set(x_3, 0, x_41); -x_4 = x_7; -goto _start; +return x_4; } else { -lean_ctor_set(x_3, 1, x_43); -lean_ctor_set(x_3, 0, x_41); -x_4 = x_7; +lean_object* x_6; lean_object* x_7; lean_object* x_8; size_t x_9; size_t x_10; lean_object* x_11; lean_object* x_12; uint64_t x_13; uint64_t x_14; uint64_t x_15; uint64_t x_16; uint64_t x_17; uint64_t x_18; uint64_t x_19; size_t x_20; size_t x_21; size_t x_22; size_t x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_6 = lean_array_uget(x_4, x_3); +x_7 = lean_unsigned_to_nat(0u); +x_8 = lean_array_uset(x_4, x_3, x_7); +x_9 = 1; +x_10 = lean_usize_add(x_3, x_9); +x_11 = lean_ctor_get(x_1, 1); +x_12 = lean_array_get_size(x_11); +x_13 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_6); +x_14 = 32; +x_15 = lean_uint64_shift_right(x_13, x_14); +x_16 = lean_uint64_xor(x_13, x_15); +x_17 = 16; +x_18 = lean_uint64_shift_right(x_16, x_17); +x_19 = lean_uint64_xor(x_16, x_18); +x_20 = lean_uint64_to_usize(x_19); +x_21 = lean_usize_of_nat(x_12); +lean_dec(x_12); +x_22 = lean_usize_sub(x_21, x_9); +x_23 = lean_usize_land(x_20, x_22); +x_24 = lean_array_uget(x_11, x_23); +x_25 = l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__3(x_6, x_6, x_24); +lean_dec(x_24); +lean_dec(x_6); +x_26 = lean_array_uset(x_8, x_3, x_25); +x_3 = x_10; +x_4 = x_26; goto _start; } } -else -{ -lean_dec(x_38); -lean_dec(x_24); -lean_free_object(x_4); -x_4 = x_7; -goto _start; } +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6) { +_start: +{ +uint8_t x_7; +x_7 = lean_usize_dec_lt(x_5, x_4); +if (x_7 == 0) +{ +lean_dec(x_1); +return x_6; } else { -lean_object* x_54; lean_object* x_55; lean_object* x_56; uint64_t x_57; uint64_t x_58; uint64_t x_59; uint64_t x_60; uint64_t x_61; size_t x_62; size_t x_63; size_t x_64; size_t x_65; lean_object* x_66; uint8_t x_67; -x_54 = lean_ctor_get(x_3, 0); -x_55 = lean_ctor_get(x_3, 1); -lean_inc(x_55); -lean_inc(x_54); -lean_dec(x_3); -x_56 = lean_array_get_size(x_55); -x_57 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_24); -x_58 = lean_uint64_shift_right(x_57, x_12); -x_59 = lean_uint64_xor(x_57, x_58); -x_60 = lean_uint64_shift_right(x_59, x_15); -x_61 = lean_uint64_xor(x_59, x_60); -x_62 = lean_uint64_to_usize(x_61); -x_63 = lean_usize_of_nat(x_56); -lean_dec(x_56); -x_64 = lean_usize_sub(x_63, x_20); -x_65 = lean_usize_land(x_62, x_64); -x_66 = lean_array_uget(x_55, x_65); -x_67 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_24, x_66); -if (x_67 == 0) +lean_object* x_8; uint8_t x_9; +x_8 = lean_array_uget(x_3, x_5); +x_9 = !lean_is_exclusive(x_6); +if (x_9 == 0) { -lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; uint8_t x_77; -x_68 = lean_unsigned_to_nat(1u); -x_69 = lean_nat_add(x_54, x_68); -lean_dec(x_54); -x_70 = lean_box(0); -lean_ctor_set(x_4, 2, x_66); -lean_ctor_set(x_4, 1, x_70); -lean_ctor_set(x_4, 0, x_24); -x_71 = lean_array_uset(x_55, x_65, x_4); -x_72 = lean_unsigned_to_nat(4u); -x_73 = lean_nat_mul(x_69, x_72); -x_74 = lean_unsigned_to_nat(3u); -x_75 = lean_nat_div(x_73, x_74); -lean_dec(x_73); -x_76 = lean_array_get_size(x_71); -x_77 = lean_nat_dec_le(x_75, x_76); -lean_dec(x_76); -lean_dec(x_75); -if (x_77 == 0) +lean_object* x_10; lean_object* x_11; lean_object* x_12; uint64_t x_13; uint64_t x_14; uint64_t x_15; uint64_t x_16; uint64_t x_17; uint64_t x_18; uint64_t x_19; size_t x_20; size_t x_21; size_t x_22; size_t x_23; size_t x_24; lean_object* x_25; uint8_t x_26; +x_10 = lean_ctor_get(x_6, 0); +x_11 = lean_ctor_get(x_6, 1); +x_12 = lean_array_get_size(x_11); +x_13 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_8); +x_14 = 32; +x_15 = lean_uint64_shift_right(x_13, x_14); +x_16 = lean_uint64_xor(x_13, x_15); +x_17 = 16; +x_18 = lean_uint64_shift_right(x_16, x_17); +x_19 = lean_uint64_xor(x_16, x_18); +x_20 = lean_uint64_to_usize(x_19); +x_21 = lean_usize_of_nat(x_12); +lean_dec(x_12); +x_22 = 1; +x_23 = lean_usize_sub(x_21, x_22); +x_24 = lean_usize_land(x_20, x_23); +x_25 = lean_array_uget(x_11, x_24); +x_26 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_8, x_25); +if (x_26 == 0) +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; +x_27 = lean_unsigned_to_nat(1u); +x_28 = lean_nat_add(x_10, x_27); +lean_dec(x_10); +x_29 = lean_box(0); +x_30 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_30, 0, x_8); +lean_ctor_set(x_30, 1, x_29); +lean_ctor_set(x_30, 2, x_25); +x_31 = lean_array_uset(x_11, x_24, x_30); +x_32 = lean_unsigned_to_nat(4u); +x_33 = lean_nat_mul(x_28, x_32); +x_34 = lean_unsigned_to_nat(3u); +x_35 = lean_nat_div(x_33, x_34); +lean_dec(x_33); +x_36 = lean_array_get_size(x_31); +x_37 = lean_nat_dec_le(x_35, x_36); +lean_dec(x_36); +lean_dec(x_35); +if (x_37 == 0) { -lean_object* x_78; lean_object* x_79; -x_78 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_71); -x_79 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_79, 0, x_69); -lean_ctor_set(x_79, 1, x_78); -x_3 = x_79; -x_4 = x_7; +lean_object* x_38; size_t x_39; +x_38 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_31); +lean_ctor_set(x_6, 1, x_38); +lean_ctor_set(x_6, 0, x_28); +x_39 = lean_usize_add(x_5, x_22); +x_5 = x_39; goto _start; } else { -lean_object* x_81; -x_81 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_81, 0, x_69); -lean_ctor_set(x_81, 1, x_71); -x_3 = x_81; -x_4 = x_7; +size_t x_41; +lean_ctor_set(x_6, 1, x_31); +lean_ctor_set(x_6, 0, x_28); +x_41 = lean_usize_add(x_5, x_22); +x_5 = x_41; goto _start; } } else { -lean_object* x_83; -lean_dec(x_66); -lean_dec(x_24); -lean_free_object(x_4); -x_83 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_83, 0, x_54); -lean_ctor_set(x_83, 1, x_55); -x_3 = x_83; -x_4 = x_7; +lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; size_t x_47; +lean_inc(x_1); +x_43 = lean_array_uset(x_11, x_24, x_1); +x_44 = lean_box(0); +x_45 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__13(x_8, x_44, x_25); +x_46 = lean_array_uset(x_43, x_24, x_45); +lean_ctor_set(x_6, 1, x_46); +x_47 = lean_usize_add(x_5, x_22); +x_5 = x_47; goto _start; } } -} else { -lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; uint64_t x_89; uint64_t x_90; uint64_t x_91; uint64_t x_92; uint64_t x_93; uint64_t x_94; uint64_t x_95; size_t x_96; size_t x_97; size_t x_98; size_t x_99; size_t x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; uint64_t x_107; uint64_t x_108; uint64_t x_109; uint64_t x_110; uint64_t x_111; size_t x_112; size_t x_113; size_t x_114; size_t x_115; lean_object* x_116; uint8_t x_117; -x_85 = lean_ctor_get(x_4, 0); -x_86 = lean_ctor_get(x_4, 2); -lean_inc(x_86); -lean_inc(x_85); -lean_dec(x_4); -x_87 = lean_ctor_get(x_2, 1); -x_88 = lean_array_get_size(x_87); -x_89 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_85); -x_90 = 32; -x_91 = lean_uint64_shift_right(x_89, x_90); -x_92 = lean_uint64_xor(x_89, x_91); -x_93 = 16; -x_94 = lean_uint64_shift_right(x_92, x_93); -x_95 = lean_uint64_xor(x_92, x_94); -x_96 = lean_uint64_to_usize(x_95); -x_97 = lean_usize_of_nat(x_88); -lean_dec(x_88); -x_98 = 1; -x_99 = lean_usize_sub(x_97, x_98); -x_100 = lean_usize_land(x_96, x_99); -x_101 = lean_array_uget(x_87, x_100); -x_102 = l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__11(x_85, x_85, x_101); -lean_dec(x_101); -lean_dec(x_85); -x_103 = lean_ctor_get(x_3, 0); -lean_inc(x_103); -x_104 = lean_ctor_get(x_3, 1); -lean_inc(x_104); -if (lean_is_exclusive(x_3)) { - lean_ctor_release(x_3, 0); - lean_ctor_release(x_3, 1); - x_105 = x_3; -} else { - lean_dec_ref(x_3); - x_105 = lean_box(0); -} -x_106 = lean_array_get_size(x_104); -x_107 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_102); -x_108 = lean_uint64_shift_right(x_107, x_90); -x_109 = lean_uint64_xor(x_107, x_108); -x_110 = lean_uint64_shift_right(x_109, x_93); -x_111 = lean_uint64_xor(x_109, x_110); -x_112 = lean_uint64_to_usize(x_111); -x_113 = lean_usize_of_nat(x_106); -lean_dec(x_106); -x_114 = lean_usize_sub(x_113, x_98); -x_115 = lean_usize_land(x_112, x_114); -x_116 = lean_array_uget(x_104, x_115); -x_117 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_102, x_116); -if (x_117 == 0) -{ -lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; uint8_t x_128; -x_118 = lean_unsigned_to_nat(1u); -x_119 = lean_nat_add(x_103, x_118); -lean_dec(x_103); -x_120 = lean_box(0); -x_121 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_121, 0, x_102); -lean_ctor_set(x_121, 1, x_120); -lean_ctor_set(x_121, 2, x_116); -x_122 = lean_array_uset(x_104, x_115, x_121); -x_123 = lean_unsigned_to_nat(4u); -x_124 = lean_nat_mul(x_119, x_123); -x_125 = lean_unsigned_to_nat(3u); -x_126 = lean_nat_div(x_124, x_125); -lean_dec(x_124); -x_127 = lean_array_get_size(x_122); -x_128 = lean_nat_dec_le(x_126, x_127); -lean_dec(x_127); -lean_dec(x_126); -if (x_128 == 0) +lean_object* x_49; lean_object* x_50; lean_object* x_51; uint64_t x_52; uint64_t x_53; uint64_t x_54; uint64_t x_55; uint64_t x_56; uint64_t x_57; uint64_t x_58; size_t x_59; size_t x_60; size_t x_61; size_t x_62; size_t x_63; lean_object* x_64; uint8_t x_65; +x_49 = lean_ctor_get(x_6, 0); +x_50 = lean_ctor_get(x_6, 1); +lean_inc(x_50); +lean_inc(x_49); +lean_dec(x_6); +x_51 = lean_array_get_size(x_50); +x_52 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_8); +x_53 = 32; +x_54 = lean_uint64_shift_right(x_52, x_53); +x_55 = lean_uint64_xor(x_52, x_54); +x_56 = 16; +x_57 = lean_uint64_shift_right(x_55, x_56); +x_58 = lean_uint64_xor(x_55, x_57); +x_59 = lean_uint64_to_usize(x_58); +x_60 = lean_usize_of_nat(x_51); +lean_dec(x_51); +x_61 = 1; +x_62 = lean_usize_sub(x_60, x_61); +x_63 = lean_usize_land(x_59, x_62); +x_64 = lean_array_uget(x_50, x_63); +x_65 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_8, x_64); +if (x_65 == 0) +{ +lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; uint8_t x_76; +x_66 = lean_unsigned_to_nat(1u); +x_67 = lean_nat_add(x_49, x_66); +lean_dec(x_49); +x_68 = lean_box(0); +x_69 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_69, 0, x_8); +lean_ctor_set(x_69, 1, x_68); +lean_ctor_set(x_69, 2, x_64); +x_70 = lean_array_uset(x_50, x_63, x_69); +x_71 = lean_unsigned_to_nat(4u); +x_72 = lean_nat_mul(x_67, x_71); +x_73 = lean_unsigned_to_nat(3u); +x_74 = lean_nat_div(x_72, x_73); +lean_dec(x_72); +x_75 = lean_array_get_size(x_70); +x_76 = lean_nat_dec_le(x_74, x_75); +lean_dec(x_75); +lean_dec(x_74); +if (x_76 == 0) { -lean_object* x_129; lean_object* x_130; -x_129 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_122); -if (lean_is_scalar(x_105)) { - x_130 = lean_alloc_ctor(0, 2, 0); -} else { - x_130 = x_105; -} -lean_ctor_set(x_130, 0, x_119); -lean_ctor_set(x_130, 1, x_129); -x_3 = x_130; -x_4 = x_86; +lean_object* x_77; lean_object* x_78; size_t x_79; +x_77 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_70); +x_78 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_78, 0, x_67); +lean_ctor_set(x_78, 1, x_77); +x_79 = lean_usize_add(x_5, x_61); +x_5 = x_79; +x_6 = x_78; goto _start; } else { -lean_object* x_132; -if (lean_is_scalar(x_105)) { - x_132 = lean_alloc_ctor(0, 2, 0); -} else { - x_132 = x_105; -} -lean_ctor_set(x_132, 0, x_119); -lean_ctor_set(x_132, 1, x_122); -x_3 = x_132; -x_4 = x_86; +lean_object* x_81; size_t x_82; +x_81 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_81, 0, x_67); +lean_ctor_set(x_81, 1, x_70); +x_82 = lean_usize_add(x_5, x_61); +x_5 = x_82; +x_6 = x_81; goto _start; } } else { -lean_object* x_134; -lean_dec(x_116); -lean_dec(x_102); -if (lean_is_scalar(x_105)) { - x_134 = lean_alloc_ctor(0, 2, 0); -} else { - x_134 = x_105; -} -lean_ctor_set(x_134, 0, x_103); -lean_ctor_set(x_134, 1, x_104); -x_3 = x_134; -x_4 = x_86; +lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; size_t x_89; +lean_inc(x_1); +x_84 = lean_array_uset(x_50, x_63, x_1); +x_85 = lean_box(0); +x_86 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__13(x_8, x_85, x_64); +x_87 = lean_array_uset(x_84, x_63, x_86); +x_88 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_88, 0, x_49); +lean_ctor_set(x_88, 1, x_87); +x_89 = lean_usize_add(x_5, x_61); +x_5 = x_89; +x_6 = x_88; goto _start; } } } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__14(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6) { -_start: -{ -uint8_t x_7; -x_7 = lean_usize_dec_eq(x_4, x_5); -if (x_7 == 0) -{ -lean_object* x_8; lean_object* x_9; size_t x_10; size_t x_11; -x_8 = lean_array_uget(x_3, x_4); -x_9 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__13(x_1, x_2, x_6, x_8); -x_10 = 1; -x_11 = lean_usize_add(x_4, x_10); -x_4 = x_11; -x_6 = x_9; -goto _start; -} -else -{ -return x_6; -} -} -} -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___lambda__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___lambda__1(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; @@ -15677,14 +17532,14 @@ return x_9; } } } -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; lean_object* x_8; lean_object* x_9; x_7 = lean_ctor_get(x_6, 2); lean_inc(x_7); lean_dec(x_6); -x_8 = lean_alloc_closure((void*)(l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___lambda__1___boxed), 2, 1); +x_8 = lean_alloc_closure((void*)(l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___lambda__1___boxed), 2, 1); lean_closure_set(x_8, 0, x_1); x_9 = l_Lean_Syntax_findStack_x3f(x_7, x_2, x_8); if (lean_obj_tag(x_9) == 0) @@ -15741,7 +17596,7 @@ return x_20; } } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, size_t x_7, size_t x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, size_t x_7, size_t x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { uint8_t x_12; @@ -15753,7 +17608,7 @@ x_13 = lean_array_uget(x_6, x_7); lean_inc(x_10); lean_inc(x_9); lean_inc(x_2); -x_14 = l_Lean_Linter_collectMacroExpansions_x3f___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__4(x_2, x_13, x_9, x_10, x_11); +x_14 = l_Lean_Linter_collectMacroExpansions_x3f___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5(x_2, x_13, x_9, x_10, x_11); if (lean_obj_tag(x_14) == 0) { lean_object* x_15; @@ -15789,7 +17644,7 @@ lean_inc(x_3); lean_inc(x_1); lean_inc(x_5); lean_inc(x_2); -x_24 = lean_alloc_closure((void*)(l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___lambda__2___boxed), 6, 5); +x_24 = lean_alloc_closure((void*)(l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___lambda__2___boxed), 6, 5); lean_closure_set(x_24, 0, x_2); lean_closure_set(x_24, 1, x_5); lean_closure_set(x_24, 2, x_1); @@ -15836,7 +17691,7 @@ lean_inc(x_3); lean_inc(x_1); lean_inc(x_5); lean_inc(x_2); -x_33 = lean_alloc_closure((void*)(l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___lambda__2___boxed), 6, 5); +x_33 = lean_alloc_closure((void*)(l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___lambda__2___boxed), 6, 5); lean_closure_set(x_33, 0, x_2); lean_closure_set(x_33, 1, x_5); lean_closure_set(x_33, 2, x_1); @@ -15921,7 +17776,7 @@ return x_47; } } } -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16___lambda__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___lambda__1(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; @@ -15945,12 +17800,12 @@ return x_7; } } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, size_t x_7, size_t x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, size_t x_7, size_t x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { lean_object* x_12; uint8_t x_13; lean_inc(x_1); -x_12 = lean_alloc_closure((void*)(l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16___lambda__1___boxed), 2, 1); +x_12 = lean_alloc_closure((void*)(l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___lambda__1___boxed), 2, 1); lean_closure_set(x_12, 0, x_1); x_13 = lean_usize_dec_eq(x_7, x_8); if (x_13 == 0) @@ -15960,7 +17815,7 @@ x_14 = lean_array_uget(x_6, x_7); lean_inc(x_10); lean_inc(x_9); lean_inc(x_3); -x_15 = l_Lean_Linter_collectMacroExpansions_x3f___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__4(x_3, x_14, x_9, x_10, x_11); +x_15 = l_Lean_Linter_collectMacroExpansions_x3f___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5(x_3, x_14, x_9, x_10, x_11); if (lean_obj_tag(x_15) == 0) { lean_object* x_16; @@ -15996,7 +17851,7 @@ lean_inc(x_5); lean_inc(x_4); lean_inc(x_2); lean_inc(x_3); -x_25 = lean_alloc_closure((void*)(l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___lambda__2___boxed), 6, 5); +x_25 = lean_alloc_closure((void*)(l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___lambda__2___boxed), 6, 5); lean_closure_set(x_25, 0, x_3); lean_closure_set(x_25, 1, x_12); lean_closure_set(x_25, 2, x_2); @@ -16042,7 +17897,7 @@ lean_inc(x_5); lean_inc(x_4); lean_inc(x_2); lean_inc(x_3); -x_34 = lean_alloc_closure((void*)(l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___lambda__2___boxed), 6, 5); +x_34 = lean_alloc_closure((void*)(l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___lambda__2___boxed), 6, 5); lean_closure_set(x_34, 0, x_3); lean_closure_set(x_34, 1, x_12); lean_closure_set(x_34, 2, x_2); @@ -16129,7 +17984,7 @@ return x_48; } } } -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__17(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6) { +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__23(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6) { _start: { uint8_t x_7; @@ -16173,7 +18028,7 @@ return x_15; } } } -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__18(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6) { +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__24(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6) { _start: { uint8_t x_7; @@ -16198,7 +18053,7 @@ x_20 = 1; x_21 = lean_usize_sub(x_19, x_20); x_22 = lean_usize_land(x_18, x_21); x_23 = lean_array_uget(x_9, x_22); -x_24 = l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__11(x_8, x_8, x_23); +x_24 = l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__3(x_8, x_8, x_23); lean_dec(x_23); lean_dec(x_8); x_25 = lean_ctor_get(x_3, 1); @@ -16239,7 +18094,7 @@ return x_41; } } } -LEAN_EXPORT uint8_t l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__1(lean_object* x_1) { +LEAN_EXPORT uint8_t l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__1(lean_object* x_1) { _start: { uint8_t x_2; @@ -16258,7 +18113,7 @@ return x_4; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__2(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__2(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; @@ -16278,218 +18133,251 @@ lean_ctor_set(x_14, 1, x_8); return x_14; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, uint8_t x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +static size_t _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__3___closed__1() { _start: { -if (x_10 == 0) +lean_object* x_1; size_t x_2; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379____closed__1; +x_2 = lean_array_size(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, uint8_t x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { +_start: { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_16 = lean_box(0); -x_17 = lean_mk_array(x_3, x_16); -x_18 = lean_unsigned_to_nat(0u); -x_19 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_19, 0, x_18); -lean_ctor_set(x_19, 1, x_17); -x_20 = lean_st_mk_ref(x_19, x_15); -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_20, 1); -lean_inc(x_22); -if (lean_is_exclusive(x_20)) { - lean_ctor_release(x_20, 0); - lean_ctor_release(x_20, 1); - x_23 = x_20; +if (x_12 == 0) +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_18 = lean_box(0); +x_19 = lean_mk_array(x_3, x_18); +x_20 = lean_unsigned_to_nat(0u); +x_21 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_21, 0, x_20); +lean_ctor_set(x_21, 1, x_19); +x_22 = lean_st_mk_ref(x_21, x_17); +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +if (lean_is_exclusive(x_22)) { + lean_ctor_release(x_22, 0); + lean_ctor_release(x_22, 1); + x_25 = x_22; } else { - lean_dec_ref(x_20); - x_23 = lean_box(0); + lean_dec_ref(x_22); + x_25 = lean_box(0); } -x_24 = lean_ctor_get(x_4, 4); +x_26 = lean_ctor_get(x_4, 4); lean_inc(x_5); -x_25 = l_Lean_Linter_UnusedVariables_visitAssignments(x_21, x_5, x_24, x_22); -lean_dec(x_21); -if (lean_obj_tag(x_25) == 0) +x_27 = l_Lean_Linter_UnusedVariables_visitAssignments(x_23, x_5, x_26, x_24); +lean_dec(x_23); +if (lean_obj_tag(x_27) == 0) { -lean_object* x_26; lean_object* x_27; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; uint8_t x_71; -x_26 = lean_ctor_get(x_25, 1); -lean_inc(x_26); -lean_dec(x_25); -x_66 = lean_st_ref_take(x_5, x_26); -x_67 = lean_ctor_get(x_66, 0); -lean_inc(x_67); -x_68 = lean_ctor_get(x_66, 1); -lean_inc(x_68); -lean_dec(x_66); -x_69 = lean_ctor_get(x_67, 1); +lean_object* x_28; lean_object* x_29; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; uint8_t x_73; size_t x_74; +x_28 = lean_ctor_get(x_27, 1); +lean_inc(x_28); +lean_dec(x_27); +x_68 = lean_st_ref_take(x_5, x_28); +x_69 = lean_ctor_get(x_68, 0); lean_inc(x_69); -lean_dec(x_67); -x_70 = lean_array_get_size(x_69); -x_71 = lean_nat_dec_lt(x_18, x_70); -if (x_71 == 0) -{ -lean_object* x_72; lean_object* x_73; -lean_dec(x_70); +x_70 = lean_ctor_get(x_68, 1); +lean_inc(x_70); +lean_dec(x_68); +x_71 = lean_ctor_get(x_69, 1); +lean_inc(x_71); lean_dec(x_69); -x_72 = lean_st_ref_set(x_5, x_9, x_68); -x_73 = lean_ctor_get(x_72, 1); -lean_inc(x_73); +x_72 = lean_array_get_size(x_71); +x_73 = lean_nat_dec_lt(x_20, x_72); +x_74 = 0; +if (x_73 == 0) +{ +size_t x_75; lean_object* x_76; lean_object* x_77; size_t x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_dec(x_72); -x_27 = x_73; -goto block_65; +lean_dec(x_71); +x_75 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__3___closed__1; +x_76 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379____closed__1; +x_77 = l_Array_mapMUnsafe_map___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__14(x_9, x_75, x_74, x_76); +x_78 = lean_array_size(x_77); +lean_inc(x_11); +x_79 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15(x_10, x_11, x_77, x_78, x_74, x_11); +lean_dec(x_77); +lean_dec(x_11); +x_80 = lean_st_ref_set(x_5, x_79, x_70); +x_81 = lean_ctor_get(x_80, 1); +lean_inc(x_81); +lean_dec(x_80); +x_29 = x_81; +goto block_67; } else { -uint8_t x_74; -x_74 = lean_nat_dec_le(x_70, x_70); -if (x_74 == 0) +uint8_t x_82; +x_82 = lean_nat_dec_le(x_72, x_72); +if (x_82 == 0) { -lean_object* x_75; lean_object* x_76; -lean_dec(x_70); -lean_dec(x_69); -x_75 = lean_st_ref_set(x_5, x_9, x_68); -x_76 = lean_ctor_get(x_75, 1); -lean_inc(x_76); -lean_dec(x_75); -x_27 = x_76; -goto block_65; +size_t x_83; lean_object* x_84; lean_object* x_85; size_t x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; +lean_dec(x_72); +lean_dec(x_71); +x_83 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__3___closed__1; +x_84 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379____closed__1; +x_85 = l_Array_mapMUnsafe_map___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16(x_9, x_83, x_74, x_84); +x_86 = lean_array_size(x_85); +lean_inc(x_11); +x_87 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__17(x_10, x_11, x_85, x_86, x_74, x_11); +lean_dec(x_85); +lean_dec(x_11); +x_88 = lean_st_ref_set(x_5, x_87, x_70); +x_89 = lean_ctor_get(x_88, 1); +lean_inc(x_89); +lean_dec(x_88); +x_29 = x_89; +goto block_67; } else { -size_t x_77; size_t x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; -x_77 = 0; -x_78 = lean_usize_of_nat(x_70); -lean_dec(x_70); -x_79 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__14(x_7, x_8, x_69, x_77, x_78, x_9); -lean_dec(x_69); -x_80 = lean_st_ref_set(x_5, x_79, x_68); -x_81 = lean_ctor_get(x_80, 1); -lean_inc(x_81); -lean_dec(x_80); -x_27 = x_81; -goto block_65; +size_t x_90; lean_object* x_91; lean_object* x_92; size_t x_93; lean_object* x_94; size_t x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; +x_90 = lean_usize_of_nat(x_72); +lean_dec(x_72); +x_91 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379____closed__1; +x_92 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__18(x_71, x_74, x_90, x_91); +lean_dec(x_71); +x_93 = lean_array_size(x_92); +x_94 = l_Array_mapMUnsafe_map___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19(x_9, x_93, x_74, x_92); +x_95 = lean_array_size(x_94); +lean_inc(x_11); +x_96 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20(x_10, x_11, x_94, x_95, x_74, x_11); +lean_dec(x_94); +lean_dec(x_11); +x_97 = lean_st_ref_set(x_5, x_96, x_70); +x_98 = lean_ctor_get(x_97, 1); +lean_inc(x_98); +lean_dec(x_97); +x_29 = x_98; +goto block_67; } } -block_65: +block_67: { -lean_object* x_28; uint8_t x_29; -x_28 = lean_st_ref_get(x_5, x_27); +lean_object* x_30; uint8_t x_31; +x_30 = lean_st_ref_get(x_5, x_29); lean_dec(x_5); -x_29 = !lean_is_exclusive(x_28); -if (x_29 == 0) +x_31 = !lean_is_exclusive(x_30); +if (x_31 == 0) { -lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; -x_30 = lean_ctor_get(x_28, 0); -x_31 = lean_ctor_get(x_28, 1); -x_32 = lean_array_get_size(x_6); -x_33 = lean_nat_dec_lt(x_18, x_32); -if (x_33 == 0) +lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; +x_32 = lean_ctor_get(x_30, 0); +x_33 = lean_ctor_get(x_30, 1); +x_34 = lean_array_get_size(x_6); +x_35 = lean_nat_dec_lt(x_20, x_34); +if (x_35 == 0) { -uint8_t x_34; lean_object* x_35; lean_object* x_36; +uint8_t x_36; lean_object* x_37; lean_object* x_38; +lean_dec(x_34); +lean_free_object(x_30); lean_dec(x_32); -lean_free_object(x_28); -lean_dec(x_30); -lean_dec(x_23); -x_34 = 1; -x_35 = lean_box(0); -x_36 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__2(x_1, x_2, x_34, x_11, x_35, x_13, x_14, x_31); -return x_36; +lean_dec(x_25); +x_36 = 1; +x_37 = lean_box(0); +x_38 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__2(x_1, x_2, x_36, x_13, x_37, x_15, x_16, x_33); +return x_38; } else { -size_t x_37; size_t x_38; uint8_t x_39; -x_37 = 0; -x_38 = lean_usize_of_nat(x_32); +size_t x_39; size_t x_40; uint8_t x_41; +x_39 = 0; +x_40 = lean_usize_of_nat(x_34); +lean_dec(x_34); +x_41 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__11(x_7, x_8, x_32, x_6, x_39, x_40); lean_dec(x_32); -x_39 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__12(x_7, x_8, x_30, x_6, x_37, x_38); -lean_dec(x_30); -if (x_39 == 0) +if (x_41 == 0) { -uint8_t x_40; lean_object* x_41; lean_object* x_42; -lean_free_object(x_28); -lean_dec(x_23); -x_40 = 1; -x_41 = lean_box(0); -x_42 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__2(x_1, x_2, x_40, x_11, x_41, x_13, x_14, x_31); -return x_42; +uint8_t x_42; lean_object* x_43; lean_object* x_44; +lean_free_object(x_30); +lean_dec(x_25); +x_42 = 1; +x_43 = lean_box(0); +x_44 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__2(x_1, x_2, x_42, x_13, x_43, x_15, x_16, x_33); +return x_44; } else { -uint8_t x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; +uint8_t x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_dec(x_2); lean_dec(x_1); -x_43 = 1; -x_44 = lean_box(x_43); -if (lean_is_scalar(x_23)) { - x_45 = lean_alloc_ctor(0, 2, 0); +x_45 = 1; +x_46 = lean_box(x_45); +if (lean_is_scalar(x_25)) { + x_47 = lean_alloc_ctor(0, 2, 0); } else { - x_45 = x_23; + x_47 = x_25; } -lean_ctor_set(x_45, 0, x_44); -lean_ctor_set(x_45, 1, x_11); -x_46 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_46, 0, x_45); -lean_ctor_set(x_28, 0, x_46); -return x_28; +lean_ctor_set(x_47, 0, x_46); +lean_ctor_set(x_47, 1, x_13); +x_48 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_48, 0, x_47); +lean_ctor_set(x_30, 0, x_48); +return x_30; } } } else { -lean_object* x_47; lean_object* x_48; lean_object* x_49; uint8_t x_50; -x_47 = lean_ctor_get(x_28, 0); -x_48 = lean_ctor_get(x_28, 1); -lean_inc(x_48); -lean_inc(x_47); -lean_dec(x_28); -x_49 = lean_array_get_size(x_6); -x_50 = lean_nat_dec_lt(x_18, x_49); -if (x_50 == 0) +lean_object* x_49; lean_object* x_50; lean_object* x_51; uint8_t x_52; +x_49 = lean_ctor_get(x_30, 0); +x_50 = lean_ctor_get(x_30, 1); +lean_inc(x_50); +lean_inc(x_49); +lean_dec(x_30); +x_51 = lean_array_get_size(x_6); +x_52 = lean_nat_dec_lt(x_20, x_51); +if (x_52 == 0) { -uint8_t x_51; lean_object* x_52; lean_object* x_53; +uint8_t x_53; lean_object* x_54; lean_object* x_55; +lean_dec(x_51); lean_dec(x_49); -lean_dec(x_47); -lean_dec(x_23); -x_51 = 1; -x_52 = lean_box(0); -x_53 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__2(x_1, x_2, x_51, x_11, x_52, x_13, x_14, x_48); -return x_53; +lean_dec(x_25); +x_53 = 1; +x_54 = lean_box(0); +x_55 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__2(x_1, x_2, x_53, x_13, x_54, x_15, x_16, x_50); +return x_55; } else { -size_t x_54; size_t x_55; uint8_t x_56; -x_54 = 0; -x_55 = lean_usize_of_nat(x_49); +size_t x_56; size_t x_57; uint8_t x_58; +x_56 = 0; +x_57 = lean_usize_of_nat(x_51); +lean_dec(x_51); +x_58 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__11(x_7, x_8, x_49, x_6, x_56, x_57); lean_dec(x_49); -x_56 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__12(x_7, x_8, x_47, x_6, x_54, x_55); -lean_dec(x_47); -if (x_56 == 0) +if (x_58 == 0) { -uint8_t x_57; lean_object* x_58; lean_object* x_59; -lean_dec(x_23); -x_57 = 1; -x_58 = lean_box(0); -x_59 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__2(x_1, x_2, x_57, x_11, x_58, x_13, x_14, x_48); -return x_59; +uint8_t x_59; lean_object* x_60; lean_object* x_61; +lean_dec(x_25); +x_59 = 1; +x_60 = lean_box(0); +x_61 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__2(x_1, x_2, x_59, x_13, x_60, x_15, x_16, x_50); +return x_61; } else { -uint8_t x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; +uint8_t x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_dec(x_2); lean_dec(x_1); -x_60 = 1; -x_61 = lean_box(x_60); -if (lean_is_scalar(x_23)) { - x_62 = lean_alloc_ctor(0, 2, 0); +x_62 = 1; +x_63 = lean_box(x_62); +if (lean_is_scalar(x_25)) { + x_64 = lean_alloc_ctor(0, 2, 0); } else { - x_62 = x_23; + x_64 = x_25; } -lean_ctor_set(x_62, 0, x_61); -lean_ctor_set(x_62, 1, x_11); -x_63 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_63, 0, x_62); -x_64 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_64, 0, x_63); -lean_ctor_set(x_64, 1, x_48); -return x_64; +lean_ctor_set(x_64, 1, x_13); +x_65 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_65, 0, x_64); +x_66 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_66, 0, x_65); +lean_ctor_set(x_66, 1, x_50); +return x_66; } } } @@ -16497,417 +18385,425 @@ return x_64; } else { -uint8_t x_82; +uint8_t x_99; +lean_dec(x_13); lean_dec(x_11); -lean_dec(x_9); +lean_dec(x_10); lean_dec(x_5); lean_dec(x_2); lean_dec(x_1); -x_82 = !lean_is_exclusive(x_25); -if (x_82 == 0) +x_99 = !lean_is_exclusive(x_27); +if (x_99 == 0) { -lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; -x_83 = lean_ctor_get(x_25, 0); -x_84 = lean_ctor_get(x_13, 6); -x_85 = lean_io_error_to_string(x_83); -x_86 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_86, 0, x_85); -x_87 = l_Lean_MessageData_ofFormat(x_86); -lean_inc(x_84); -if (lean_is_scalar(x_23)) { - x_88 = lean_alloc_ctor(0, 2, 0); +lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; +x_100 = lean_ctor_get(x_27, 0); +x_101 = lean_ctor_get(x_15, 6); +x_102 = lean_io_error_to_string(x_100); +x_103 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_103, 0, x_102); +x_104 = l_Lean_MessageData_ofFormat(x_103); +lean_inc(x_101); +if (lean_is_scalar(x_25)) { + x_105 = lean_alloc_ctor(0, 2, 0); } else { - x_88 = x_23; + x_105 = x_25; } -lean_ctor_set(x_88, 0, x_84); -lean_ctor_set(x_88, 1, x_87); -lean_ctor_set(x_25, 0, x_88); -return x_25; +lean_ctor_set(x_105, 0, x_101); +lean_ctor_set(x_105, 1, x_104); +lean_ctor_set(x_27, 0, x_105); +return x_27; } else { -lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; -x_89 = lean_ctor_get(x_25, 0); -x_90 = lean_ctor_get(x_25, 1); -lean_inc(x_90); -lean_inc(x_89); -lean_dec(x_25); -x_91 = lean_ctor_get(x_13, 6); -x_92 = lean_io_error_to_string(x_89); -x_93 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_93, 0, x_92); -x_94 = l_Lean_MessageData_ofFormat(x_93); -lean_inc(x_91); -if (lean_is_scalar(x_23)) { - x_95 = lean_alloc_ctor(0, 2, 0); +lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; +x_106 = lean_ctor_get(x_27, 0); +x_107 = lean_ctor_get(x_27, 1); +lean_inc(x_107); +lean_inc(x_106); +lean_dec(x_27); +x_108 = lean_ctor_get(x_15, 6); +x_109 = lean_io_error_to_string(x_106); +x_110 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_110, 0, x_109); +x_111 = l_Lean_MessageData_ofFormat(x_110); +lean_inc(x_108); +if (lean_is_scalar(x_25)) { + x_112 = lean_alloc_ctor(0, 2, 0); } else { - x_95 = x_23; + x_112 = x_25; } -lean_ctor_set(x_95, 0, x_91); -lean_ctor_set(x_95, 1, x_94); -x_96 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_96, 0, x_95); -lean_ctor_set(x_96, 1, x_90); -return x_96; +lean_ctor_set(x_112, 0, x_108); +lean_ctor_set(x_112, 1, x_111); +x_113 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_113, 0, x_112); +lean_ctor_set(x_113, 1, x_107); +return x_113; } } } else { -lean_object* x_97; lean_object* x_98; -lean_dec(x_9); +lean_object* x_114; lean_object* x_115; +lean_dec(x_11); +lean_dec(x_10); lean_dec(x_5); lean_dec(x_3); -x_97 = lean_box(0); -x_98 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__2(x_1, x_2, x_10, x_11, x_97, x_13, x_14, x_15); -return x_98; +x_114 = lean_box(0); +x_115 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__2(x_1, x_2, x_12, x_13, x_114, x_15, x_16, x_17); +return x_115; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, uint8_t x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, uint8_t x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19, lean_object* x_20, lean_object* x_21) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, uint8_t x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, uint8_t x_18, lean_object* x_19, lean_object* x_20, lean_object* x_21, lean_object* x_22, lean_object* x_23) { _start: { -uint8_t x_22; lean_object* x_23; -if (x_10 == 0) +uint8_t x_24; lean_object* x_25; +if (x_12 == 0) { -uint8_t x_31; +uint8_t x_33; +lean_dec(x_16); +lean_dec(x_15); lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -x_31 = 0; -x_22 = x_31; -x_23 = x_21; -goto block_30; +x_33 = 0; +x_24 = x_33; +x_25 = x_23; +goto block_32; } else { -size_t x_32; size_t x_33; lean_object* x_34; -x_32 = 0; -x_33 = lean_usize_of_nat(x_11); -lean_inc(x_20); -lean_inc(x_19); +size_t x_34; size_t x_35; lean_object* x_36; +x_34 = 0; +x_35 = lean_usize_of_nat(x_13); +lean_inc(x_22); +lean_inc(x_21); lean_inc(x_1); -lean_inc(x_12); -x_34 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16(x_12, x_13, x_12, x_1, x_14, x_15, x_32, x_33, x_19, x_20, x_21); -if (lean_obj_tag(x_34) == 0) +lean_inc(x_14); +x_36 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22(x_14, x_15, x_14, x_1, x_16, x_17, x_34, x_35, x_21, x_22, x_23); +if (lean_obj_tag(x_36) == 0) { -lean_object* x_35; lean_object* x_36; uint8_t x_37; -x_35 = lean_ctor_get(x_34, 0); -lean_inc(x_35); -x_36 = lean_ctor_get(x_34, 1); -lean_inc(x_36); -lean_dec(x_34); -x_37 = lean_unbox(x_35); -lean_dec(x_35); -x_22 = x_37; -x_23 = x_36; -goto block_30; +lean_object* x_37; lean_object* x_38; uint8_t x_39; +x_37 = lean_ctor_get(x_36, 0); +lean_inc(x_37); +x_38 = lean_ctor_get(x_36, 1); +lean_inc(x_38); +lean_dec(x_36); +x_39 = lean_unbox(x_37); +lean_dec(x_37); +x_24 = x_39; +x_25 = x_38; +goto block_32; } else { -uint8_t x_38; -lean_dec(x_20); +uint8_t x_40; +lean_dec(x_22); +lean_dec(x_21); lean_dec(x_19); -lean_dec(x_17); -lean_dec(x_9); +lean_dec(x_11); +lean_dec(x_10); lean_dec(x_5); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_38 = !lean_is_exclusive(x_34); -if (x_38 == 0) +x_40 = !lean_is_exclusive(x_36); +if (x_40 == 0) { -return x_34; +return x_36; } else { -lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_39 = lean_ctor_get(x_34, 0); -x_40 = lean_ctor_get(x_34, 1); -lean_inc(x_40); -lean_inc(x_39); -lean_dec(x_34); -x_41 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_41, 0, x_39); -lean_ctor_set(x_41, 1, x_40); -return x_41; +lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_41 = lean_ctor_get(x_36, 0); +x_42 = lean_ctor_get(x_36, 1); +lean_inc(x_42); +lean_inc(x_41); +lean_dec(x_36); +x_43 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_43, 0, x_41); +lean_ctor_set(x_43, 1, x_42); +return x_43; } } } -block_30: +block_32: { -if (x_22 == 0) +if (x_24 == 0) { -lean_object* x_24; lean_object* x_25; -x_24 = lean_box(0); -x_25 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_16, x_17, x_24, x_19, x_20, x_23); -lean_dec(x_20); -lean_dec(x_19); -return x_25; +lean_object* x_26; lean_object* x_27; +x_26 = lean_box(0); +x_27 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_18, x_19, x_26, x_21, x_22, x_25); +lean_dec(x_22); +lean_dec(x_21); +return x_27; } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; -lean_dec(x_20); -lean_dec(x_19); -lean_dec(x_9); +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +lean_dec(x_22); +lean_dec(x_21); +lean_dec(x_11); +lean_dec(x_10); lean_dec(x_5); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_26 = lean_box(x_16); -x_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_26); -lean_ctor_set(x_27, 1, x_17); -x_28 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_28, 0, x_27); +x_28 = lean_box(x_18); x_29 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_29, 0, x_28); -lean_ctor_set(x_29, 1, x_23); -return x_29; +lean_ctor_set(x_29, 1, x_19); +x_30 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_30, 0, x_29); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_30); +lean_ctor_set(x_31, 1, x_25); +return x_31; } } } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__5___closed__1() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__5___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__1___boxed), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__1___boxed), 1, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, uint8_t x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, uint8_t x_17, lean_object* x_18, lean_object* x_19, lean_object* x_20, lean_object* x_21, lean_object* x_22) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, uint8_t x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, uint8_t x_19, lean_object* x_20, lean_object* x_21, lean_object* x_22, lean_object* x_23, lean_object* x_24) { _start: { -lean_object* x_23; lean_object* x_24; lean_object* x_25; +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_inc(x_1); -x_23 = lean_alloc_closure((void*)(l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16___lambda__1___boxed), 2, 1); -lean_closure_set(x_23, 0, x_1); -x_24 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__5___closed__1; -x_25 = l_Lean_Syntax_findStack_x3f(x_2, x_23, x_24); -if (lean_obj_tag(x_25) == 0) +x_25 = lean_alloc_closure((void*)(l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___lambda__1___boxed), 2, 1); +lean_closure_set(x_25, 0, x_1); +x_26 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__5___closed__1; +x_27 = l_Lean_Syntax_findStack_x3f(x_2, x_25, x_26); +if (lean_obj_tag(x_27) == 0) { -lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; -lean_dec(x_21); -lean_dec(x_20); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_11); +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +lean_dec(x_23); +lean_dec(x_22); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_13); +lean_dec(x_12); lean_dec(x_7); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_26 = lean_box(x_17); -x_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_26); -lean_ctor_set(x_27, 1, x_18); -x_28 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_28, 0, x_27); +x_28 = lean_box(x_19); x_29 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_29, 0, x_28); -lean_ctor_set(x_29, 1, x_22); -return x_29; +lean_ctor_set(x_29, 1, x_20); +x_30 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_30, 0, x_29); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_30); +lean_ctor_set(x_31, 1, x_24); +return x_31; } else { -uint8_t x_30; -x_30 = !lean_is_exclusive(x_25); -if (x_30 == 0) +uint8_t x_32; +x_32 = !lean_is_exclusive(x_27); +if (x_32 == 0) { -lean_object* x_31; -x_31 = lean_ctor_get(x_25, 0); -if (lean_obj_tag(x_31) == 0) +lean_object* x_33; +x_33 = lean_ctor_get(x_27, 0); +if (lean_obj_tag(x_33) == 0) { -lean_object* x_32; lean_object* x_33; lean_object* x_34; -lean_dec(x_21); -lean_dec(x_20); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_11); +lean_object* x_34; lean_object* x_35; lean_object* x_36; +lean_dec(x_23); +lean_dec(x_22); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_13); +lean_dec(x_12); lean_dec(x_7); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_32 = lean_box(x_17); -x_33 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_33, 0, x_32); -lean_ctor_set(x_33, 1, x_18); -lean_ctor_set(x_25, 0, x_33); -x_34 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_34, 0, x_25); -lean_ctor_set(x_34, 1, x_22); -return x_34; +x_34 = lean_box(x_19); +x_35 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_35, 0, x_34); +lean_ctor_set(x_35, 1, x_20); +lean_ctor_set(x_27, 0, x_35); +x_36 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_36, 0, x_27); +lean_ctor_set(x_36, 1, x_24); +return x_36; } else { -uint8_t x_35; -x_35 = !lean_is_exclusive(x_31); -if (x_35 == 0) -{ -lean_object* x_36; uint8_t x_37; -x_36 = lean_ctor_get(x_31, 0); -x_37 = !lean_is_exclusive(x_36); +uint8_t x_37; +x_37 = !lean_is_exclusive(x_33); if (x_37 == 0) { -lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; -x_38 = lean_ctor_get(x_31, 1); -x_39 = lean_ctor_get(x_36, 0); -x_40 = lean_ctor_get(x_36, 1); -lean_dec(x_40); -x_41 = l_Lean_Syntax_isIdent(x_39); -lean_dec(x_39); -if (x_41 == 0) +lean_object* x_38; uint8_t x_39; +x_38 = lean_ctor_get(x_33, 0); +x_39 = !lean_is_exclusive(x_38); +if (x_39 == 0) { -lean_object* x_42; lean_object* x_43; -lean_free_object(x_36); -lean_free_object(x_31); -lean_dec(x_38); -lean_free_object(x_25); -x_42 = lean_box(0); -x_43 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_1, x_14, x_15, x_16, x_17, x_18, x_42, x_20, x_21, x_22); -return x_43; +lean_object* x_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; +x_40 = lean_ctor_get(x_33, 1); +x_41 = lean_ctor_get(x_38, 0); +x_42 = lean_ctor_get(x_38, 1); +lean_dec(x_42); +x_43 = l_Lean_Syntax_isIdent(x_41); +lean_dec(x_41); +if (x_43 == 0) +{ +lean_object* x_44; lean_object* x_45; +lean_free_object(x_38); +lean_free_object(x_33); +lean_dec(x_40); +lean_free_object(x_27); +x_44 = lean_box(0); +x_45 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_1, x_16, x_17, x_18, x_19, x_20, x_44, x_22, x_23, x_24); +return x_45; } else { -lean_object* x_44; lean_object* x_45; uint8_t x_46; -x_44 = lean_array_get_size(x_14); -x_45 = lean_unsigned_to_nat(0u); -x_46 = lean_nat_dec_lt(x_45, x_44); -if (x_46 == 0) +lean_object* x_46; lean_object* x_47; uint8_t x_48; +x_46 = lean_array_get_size(x_16); +x_47 = lean_unsigned_to_nat(0u); +x_48 = lean_nat_dec_lt(x_47, x_46); +if (x_48 == 0) { -lean_object* x_47; lean_object* x_48; -lean_dec(x_44); -lean_free_object(x_36); -lean_free_object(x_31); -lean_dec(x_38); -lean_free_object(x_25); -x_47 = lean_box(0); -x_48 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_1, x_14, x_15, x_16, x_17, x_18, x_47, x_20, x_21, x_22); -return x_48; +lean_object* x_49; lean_object* x_50; +lean_dec(x_46); +lean_free_object(x_38); +lean_free_object(x_33); +lean_dec(x_40); +lean_free_object(x_27); +x_49 = lean_box(0); +x_50 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_1, x_16, x_17, x_18, x_19, x_20, x_49, x_22, x_23, x_24); +return x_50; } else { -size_t x_49; size_t x_50; uint8_t x_51; -x_49 = 0; -x_50 = lean_usize_of_nat(x_44); -lean_dec(x_44); -lean_inc(x_15); +size_t x_51; size_t x_52; uint8_t x_53; +x_51 = 0; +x_52 = lean_usize_of_nat(x_46); +lean_dec(x_46); +lean_inc(x_17); lean_inc(x_3); -x_51 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__17(x_3, x_15, x_38, x_14, x_49, x_50); -if (x_51 == 0) -{ -lean_object* x_52; lean_object* x_53; -lean_free_object(x_36); -lean_free_object(x_31); -lean_free_object(x_25); -x_52 = lean_box(0); -x_53 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_1, x_14, x_15, x_16, x_17, x_18, x_52, x_20, x_21, x_22); -return x_53; +x_53 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__23(x_3, x_17, x_40, x_16, x_51, x_52); +if (x_53 == 0) +{ +lean_object* x_54; lean_object* x_55; +lean_free_object(x_38); +lean_free_object(x_33); +lean_free_object(x_27); +x_54 = lean_box(0); +x_55 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_1, x_16, x_17, x_18, x_19, x_20, x_54, x_22, x_23, x_24); +return x_55; } else { -lean_object* x_54; -lean_dec(x_21); -lean_dec(x_20); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_11); +lean_object* x_56; +lean_dec(x_23); +lean_dec(x_22); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_13); +lean_dec(x_12); lean_dec(x_7); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_54 = lean_box(x_17); -lean_ctor_set(x_36, 1, x_18); -lean_ctor_set(x_36, 0, x_54); -lean_ctor_set(x_25, 0, x_36); -lean_ctor_set_tag(x_31, 0); -lean_ctor_set(x_31, 1, x_22); -lean_ctor_set(x_31, 0, x_25); -return x_31; +x_56 = lean_box(x_19); +lean_ctor_set(x_38, 1, x_20); +lean_ctor_set(x_38, 0, x_56); +lean_ctor_set(x_27, 0, x_38); +lean_ctor_set_tag(x_33, 0); +lean_ctor_set(x_33, 1, x_24); +lean_ctor_set(x_33, 0, x_27); +return x_33; } } } } else { -lean_object* x_55; lean_object* x_56; uint8_t x_57; -x_55 = lean_ctor_get(x_31, 1); -x_56 = lean_ctor_get(x_36, 0); -lean_inc(x_56); -lean_dec(x_36); -x_57 = l_Lean_Syntax_isIdent(x_56); -lean_dec(x_56); -if (x_57 == 0) +lean_object* x_57; lean_object* x_58; uint8_t x_59; +x_57 = lean_ctor_get(x_33, 1); +x_58 = lean_ctor_get(x_38, 0); +lean_inc(x_58); +lean_dec(x_38); +x_59 = l_Lean_Syntax_isIdent(x_58); +lean_dec(x_58); +if (x_59 == 0) { -lean_object* x_58; lean_object* x_59; -lean_free_object(x_31); -lean_dec(x_55); -lean_free_object(x_25); -x_58 = lean_box(0); -x_59 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_1, x_14, x_15, x_16, x_17, x_18, x_58, x_20, x_21, x_22); -return x_59; +lean_object* x_60; lean_object* x_61; +lean_free_object(x_33); +lean_dec(x_57); +lean_free_object(x_27); +x_60 = lean_box(0); +x_61 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_1, x_16, x_17, x_18, x_19, x_20, x_60, x_22, x_23, x_24); +return x_61; } else { -lean_object* x_60; lean_object* x_61; uint8_t x_62; -x_60 = lean_array_get_size(x_14); -x_61 = lean_unsigned_to_nat(0u); -x_62 = lean_nat_dec_lt(x_61, x_60); -if (x_62 == 0) +lean_object* x_62; lean_object* x_63; uint8_t x_64; +x_62 = lean_array_get_size(x_16); +x_63 = lean_unsigned_to_nat(0u); +x_64 = lean_nat_dec_lt(x_63, x_62); +if (x_64 == 0) { -lean_object* x_63; lean_object* x_64; -lean_dec(x_60); -lean_free_object(x_31); -lean_dec(x_55); -lean_free_object(x_25); -x_63 = lean_box(0); -x_64 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_1, x_14, x_15, x_16, x_17, x_18, x_63, x_20, x_21, x_22); -return x_64; +lean_object* x_65; lean_object* x_66; +lean_dec(x_62); +lean_free_object(x_33); +lean_dec(x_57); +lean_free_object(x_27); +x_65 = lean_box(0); +x_66 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_1, x_16, x_17, x_18, x_19, x_20, x_65, x_22, x_23, x_24); +return x_66; } else { -size_t x_65; size_t x_66; uint8_t x_67; -x_65 = 0; -x_66 = lean_usize_of_nat(x_60); -lean_dec(x_60); -lean_inc(x_15); +size_t x_67; size_t x_68; uint8_t x_69; +x_67 = 0; +x_68 = lean_usize_of_nat(x_62); +lean_dec(x_62); +lean_inc(x_17); lean_inc(x_3); -x_67 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__17(x_3, x_15, x_55, x_14, x_65, x_66); -if (x_67 == 0) +x_69 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__23(x_3, x_17, x_57, x_16, x_67, x_68); +if (x_69 == 0) { -lean_object* x_68; lean_object* x_69; -lean_free_object(x_31); -lean_free_object(x_25); -x_68 = lean_box(0); -x_69 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_1, x_14, x_15, x_16, x_17, x_18, x_68, x_20, x_21, x_22); -return x_69; +lean_object* x_70; lean_object* x_71; +lean_free_object(x_33); +lean_free_object(x_27); +x_70 = lean_box(0); +x_71 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_1, x_16, x_17, x_18, x_19, x_20, x_70, x_22, x_23, x_24); +return x_71; } else { -lean_object* x_70; lean_object* x_71; -lean_dec(x_21); -lean_dec(x_20); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_11); +lean_object* x_72; lean_object* x_73; +lean_dec(x_23); +lean_dec(x_22); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_13); +lean_dec(x_12); lean_dec(x_7); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_70 = lean_box(x_17); -x_71 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_71, 0, x_70); -lean_ctor_set(x_71, 1, x_18); -lean_ctor_set(x_25, 0, x_71); -lean_ctor_set_tag(x_31, 0); -lean_ctor_set(x_31, 1, x_22); -lean_ctor_set(x_31, 0, x_25); -return x_31; +x_72 = lean_box(x_19); +x_73 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_73, 0, x_72); +lean_ctor_set(x_73, 1, x_20); +lean_ctor_set(x_27, 0, x_73); +lean_ctor_set_tag(x_33, 0); +lean_ctor_set(x_33, 1, x_24); +lean_ctor_set(x_33, 0, x_27); +return x_33; } } } @@ -16915,95 +18811,96 @@ return x_31; } else { -lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; uint8_t x_76; -x_72 = lean_ctor_get(x_31, 0); -x_73 = lean_ctor_get(x_31, 1); -lean_inc(x_73); -lean_inc(x_72); -lean_dec(x_31); -x_74 = lean_ctor_get(x_72, 0); +lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; uint8_t x_78; +x_74 = lean_ctor_get(x_33, 0); +x_75 = lean_ctor_get(x_33, 1); +lean_inc(x_75); lean_inc(x_74); -if (lean_is_exclusive(x_72)) { - lean_ctor_release(x_72, 0); - lean_ctor_release(x_72, 1); - x_75 = x_72; +lean_dec(x_33); +x_76 = lean_ctor_get(x_74, 0); +lean_inc(x_76); +if (lean_is_exclusive(x_74)) { + lean_ctor_release(x_74, 0); + lean_ctor_release(x_74, 1); + x_77 = x_74; } else { - lean_dec_ref(x_72); - x_75 = lean_box(0); + lean_dec_ref(x_74); + x_77 = lean_box(0); } -x_76 = l_Lean_Syntax_isIdent(x_74); -lean_dec(x_74); -if (x_76 == 0) +x_78 = l_Lean_Syntax_isIdent(x_76); +lean_dec(x_76); +if (x_78 == 0) { -lean_object* x_77; lean_object* x_78; +lean_object* x_79; lean_object* x_80; +lean_dec(x_77); lean_dec(x_75); -lean_dec(x_73); -lean_free_object(x_25); -x_77 = lean_box(0); -x_78 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_1, x_14, x_15, x_16, x_17, x_18, x_77, x_20, x_21, x_22); -return x_78; +lean_free_object(x_27); +x_79 = lean_box(0); +x_80 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_1, x_16, x_17, x_18, x_19, x_20, x_79, x_22, x_23, x_24); +return x_80; } else { -lean_object* x_79; lean_object* x_80; uint8_t x_81; -x_79 = lean_array_get_size(x_14); -x_80 = lean_unsigned_to_nat(0u); -x_81 = lean_nat_dec_lt(x_80, x_79); -if (x_81 == 0) +lean_object* x_81; lean_object* x_82; uint8_t x_83; +x_81 = lean_array_get_size(x_16); +x_82 = lean_unsigned_to_nat(0u); +x_83 = lean_nat_dec_lt(x_82, x_81); +if (x_83 == 0) { -lean_object* x_82; lean_object* x_83; -lean_dec(x_79); +lean_object* x_84; lean_object* x_85; +lean_dec(x_81); +lean_dec(x_77); lean_dec(x_75); -lean_dec(x_73); -lean_free_object(x_25); -x_82 = lean_box(0); -x_83 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_1, x_14, x_15, x_16, x_17, x_18, x_82, x_20, x_21, x_22); -return x_83; +lean_free_object(x_27); +x_84 = lean_box(0); +x_85 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_1, x_16, x_17, x_18, x_19, x_20, x_84, x_22, x_23, x_24); +return x_85; } else { -size_t x_84; size_t x_85; uint8_t x_86; -x_84 = 0; -x_85 = lean_usize_of_nat(x_79); -lean_dec(x_79); -lean_inc(x_15); +size_t x_86; size_t x_87; uint8_t x_88; +x_86 = 0; +x_87 = lean_usize_of_nat(x_81); +lean_dec(x_81); +lean_inc(x_17); lean_inc(x_3); -x_86 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__17(x_3, x_15, x_73, x_14, x_84, x_85); -if (x_86 == 0) +x_88 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__23(x_3, x_17, x_75, x_16, x_86, x_87); +if (x_88 == 0) { -lean_object* x_87; lean_object* x_88; -lean_dec(x_75); -lean_free_object(x_25); -x_87 = lean_box(0); -x_88 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_1, x_14, x_15, x_16, x_17, x_18, x_87, x_20, x_21, x_22); -return x_88; +lean_object* x_89; lean_object* x_90; +lean_dec(x_77); +lean_free_object(x_27); +x_89 = lean_box(0); +x_90 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_1, x_16, x_17, x_18, x_19, x_20, x_89, x_22, x_23, x_24); +return x_90; } else { -lean_object* x_89; lean_object* x_90; lean_object* x_91; -lean_dec(x_21); -lean_dec(x_20); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_11); +lean_object* x_91; lean_object* x_92; lean_object* x_93; +lean_dec(x_23); +lean_dec(x_22); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_13); +lean_dec(x_12); lean_dec(x_7); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_89 = lean_box(x_17); -if (lean_is_scalar(x_75)) { - x_90 = lean_alloc_ctor(0, 2, 0); +x_91 = lean_box(x_19); +if (lean_is_scalar(x_77)) { + x_92 = lean_alloc_ctor(0, 2, 0); } else { - x_90 = x_75; + x_92 = x_77; } -lean_ctor_set(x_90, 0, x_89); -lean_ctor_set(x_90, 1, x_18); -lean_ctor_set(x_25, 0, x_90); -x_91 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_91, 0, x_25); -lean_ctor_set(x_91, 1, x_22); -return x_91; +lean_ctor_set(x_92, 0, x_91); +lean_ctor_set(x_92, 1, x_20); +lean_ctor_set(x_27, 0, x_92); +x_93 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_93, 0, x_27); +lean_ctor_set(x_93, 1, x_24); +return x_93; } } } @@ -17012,139 +18909,140 @@ return x_91; } else { -lean_object* x_92; -x_92 = lean_ctor_get(x_25, 0); -lean_inc(x_92); -lean_dec(x_25); -if (lean_obj_tag(x_92) == 0) +lean_object* x_94; +x_94 = lean_ctor_get(x_27, 0); +lean_inc(x_94); +lean_dec(x_27); +if (lean_obj_tag(x_94) == 0) { -lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; -lean_dec(x_21); -lean_dec(x_20); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_11); +lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; +lean_dec(x_23); +lean_dec(x_22); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_13); +lean_dec(x_12); lean_dec(x_7); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_93 = lean_box(x_17); -x_94 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_94, 0, x_93); -lean_ctor_set(x_94, 1, x_18); -x_95 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_95, 0, x_94); +x_95 = lean_box(x_19); x_96 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_96, 0, x_95); -lean_ctor_set(x_96, 1, x_22); -return x_96; +lean_ctor_set(x_96, 1, x_20); +x_97 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_97, 0, x_96); +x_98 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_98, 0, x_97); +lean_ctor_set(x_98, 1, x_24); +return x_98; } else { -lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; uint8_t x_102; -x_97 = lean_ctor_get(x_92, 0); -lean_inc(x_97); -x_98 = lean_ctor_get(x_92, 1); -lean_inc(x_98); -if (lean_is_exclusive(x_92)) { - lean_ctor_release(x_92, 0); - lean_ctor_release(x_92, 1); - x_99 = x_92; -} else { - lean_dec_ref(x_92); - x_99 = lean_box(0); -} -x_100 = lean_ctor_get(x_97, 0); +lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; uint8_t x_104; +x_99 = lean_ctor_get(x_94, 0); +lean_inc(x_99); +x_100 = lean_ctor_get(x_94, 1); lean_inc(x_100); -if (lean_is_exclusive(x_97)) { - lean_ctor_release(x_97, 0); - lean_ctor_release(x_97, 1); - x_101 = x_97; +if (lean_is_exclusive(x_94)) { + lean_ctor_release(x_94, 0); + lean_ctor_release(x_94, 1); + x_101 = x_94; } else { - lean_dec_ref(x_97); + lean_dec_ref(x_94); x_101 = lean_box(0); } -x_102 = l_Lean_Syntax_isIdent(x_100); -lean_dec(x_100); -if (x_102 == 0) +x_102 = lean_ctor_get(x_99, 0); +lean_inc(x_102); +if (lean_is_exclusive(x_99)) { + lean_ctor_release(x_99, 0); + lean_ctor_release(x_99, 1); + x_103 = x_99; +} else { + lean_dec_ref(x_99); + x_103 = lean_box(0); +} +x_104 = l_Lean_Syntax_isIdent(x_102); +lean_dec(x_102); +if (x_104 == 0) { -lean_object* x_103; lean_object* x_104; +lean_object* x_105; lean_object* x_106; +lean_dec(x_103); lean_dec(x_101); -lean_dec(x_99); -lean_dec(x_98); -x_103 = lean_box(0); -x_104 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_1, x_14, x_15, x_16, x_17, x_18, x_103, x_20, x_21, x_22); -return x_104; +lean_dec(x_100); +x_105 = lean_box(0); +x_106 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_1, x_16, x_17, x_18, x_19, x_20, x_105, x_22, x_23, x_24); +return x_106; } else { -lean_object* x_105; lean_object* x_106; uint8_t x_107; -x_105 = lean_array_get_size(x_14); -x_106 = lean_unsigned_to_nat(0u); -x_107 = lean_nat_dec_lt(x_106, x_105); -if (x_107 == 0) +lean_object* x_107; lean_object* x_108; uint8_t x_109; +x_107 = lean_array_get_size(x_16); +x_108 = lean_unsigned_to_nat(0u); +x_109 = lean_nat_dec_lt(x_108, x_107); +if (x_109 == 0) { -lean_object* x_108; lean_object* x_109; -lean_dec(x_105); +lean_object* x_110; lean_object* x_111; +lean_dec(x_107); +lean_dec(x_103); lean_dec(x_101); -lean_dec(x_99); -lean_dec(x_98); -x_108 = lean_box(0); -x_109 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_1, x_14, x_15, x_16, x_17, x_18, x_108, x_20, x_21, x_22); -return x_109; +lean_dec(x_100); +x_110 = lean_box(0); +x_111 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_1, x_16, x_17, x_18, x_19, x_20, x_110, x_22, x_23, x_24); +return x_111; } else { -size_t x_110; size_t x_111; uint8_t x_112; -x_110 = 0; -x_111 = lean_usize_of_nat(x_105); -lean_dec(x_105); -lean_inc(x_15); +size_t x_112; size_t x_113; uint8_t x_114; +x_112 = 0; +x_113 = lean_usize_of_nat(x_107); +lean_dec(x_107); +lean_inc(x_17); lean_inc(x_3); -x_112 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__17(x_3, x_15, x_98, x_14, x_110, x_111); -if (x_112 == 0) +x_114 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__23(x_3, x_17, x_100, x_16, x_112, x_113); +if (x_114 == 0) { -lean_object* x_113; lean_object* x_114; +lean_object* x_115; lean_object* x_116; +lean_dec(x_103); lean_dec(x_101); -lean_dec(x_99); -x_113 = lean_box(0); -x_114 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_1, x_14, x_15, x_16, x_17, x_18, x_113, x_20, x_21, x_22); -return x_114; +x_115 = lean_box(0); +x_116 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_1, x_16, x_17, x_18, x_19, x_20, x_115, x_22, x_23, x_24); +return x_116; } else { -lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; -lean_dec(x_21); -lean_dec(x_20); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_11); +lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; +lean_dec(x_23); +lean_dec(x_22); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_13); +lean_dec(x_12); lean_dec(x_7); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_115 = lean_box(x_17); -if (lean_is_scalar(x_101)) { - x_116 = lean_alloc_ctor(0, 2, 0); -} else { - x_116 = x_101; -} -lean_ctor_set(x_116, 0, x_115); -lean_ctor_set(x_116, 1, x_18); -x_117 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_117, 0, x_116); -if (lean_is_scalar(x_99)) { +x_117 = lean_box(x_19); +if (lean_is_scalar(x_103)) { x_118 = lean_alloc_ctor(0, 2, 0); } else { - x_118 = x_99; - lean_ctor_set_tag(x_118, 0); + x_118 = x_103; } lean_ctor_set(x_118, 0, x_117); -lean_ctor_set(x_118, 1, x_22); -return x_118; +lean_ctor_set(x_118, 1, x_20); +x_119 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_119, 0, x_118); +if (lean_is_scalar(x_101)) { + x_120 = lean_alloc_ctor(0, 2, 0); +} else { + x_120 = x_101; + lean_ctor_set_tag(x_120, 0); } +lean_ctor_set(x_120, 0, x_119); +lean_ctor_set(x_120, 1, x_24); +return x_120; } } } @@ -17152,54 +19050,56 @@ return x_118; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, uint8_t x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, uint8_t x_17, lean_object* x_18, lean_object* x_19, lean_object* x_20, lean_object* x_21, lean_object* x_22) { +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, uint8_t x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, uint8_t x_19, lean_object* x_20, lean_object* x_21, lean_object* x_22, lean_object* x_23, lean_object* x_24) { _start: { -lean_object* x_23; uint8_t x_24; -x_23 = lean_ctor_get(x_6, 0); -lean_inc(x_23); -x_24 = !lean_is_exclusive(x_23); -if (x_24 == 0) +lean_object* x_25; uint8_t x_26; +x_25 = lean_ctor_get(x_6, 0); +lean_inc(x_25); +x_26 = !lean_is_exclusive(x_25); +if (x_26 == 0) { -lean_object* x_25; lean_object* x_26; lean_object* x_27; uint64_t x_28; uint64_t x_29; uint64_t x_30; uint64_t x_31; uint64_t x_32; uint64_t x_33; uint64_t x_34; size_t x_35; size_t x_36; size_t x_37; size_t x_38; size_t x_39; lean_object* x_40; uint8_t x_41; -x_25 = lean_ctor_get(x_23, 1); -x_26 = lean_ctor_get(x_23, 0); -lean_dec(x_26); -x_27 = lean_array_get_size(x_25); -x_28 = l___private_Lean_Syntax_0__String_hashRange____x40_Lean_Syntax___hyg_169_(x_1); -x_29 = 32; -x_30 = lean_uint64_shift_right(x_28, x_29); -x_31 = lean_uint64_xor(x_28, x_30); -x_32 = 16; -x_33 = lean_uint64_shift_right(x_31, x_32); -x_34 = lean_uint64_xor(x_31, x_33); -x_35 = lean_uint64_to_usize(x_34); -x_36 = lean_usize_of_nat(x_27); +lean_object* x_27; lean_object* x_28; lean_object* x_29; uint64_t x_30; uint64_t x_31; uint64_t x_32; uint64_t x_33; uint64_t x_34; uint64_t x_35; uint64_t x_36; size_t x_37; size_t x_38; size_t x_39; size_t x_40; size_t x_41; lean_object* x_42; uint8_t x_43; +x_27 = lean_ctor_get(x_25, 1); +x_28 = lean_ctor_get(x_25, 0); +lean_dec(x_28); +x_29 = lean_array_get_size(x_27); +x_30 = l___private_Lean_Syntax_0__String_hashRange____x40_Lean_Syntax___hyg_169_(x_1); +x_31 = 32; +x_32 = lean_uint64_shift_right(x_30, x_31); +x_33 = lean_uint64_xor(x_30, x_32); +x_34 = 16; +x_35 = lean_uint64_shift_right(x_33, x_34); +x_36 = lean_uint64_xor(x_33, x_35); +x_37 = lean_uint64_to_usize(x_36); +x_38 = lean_usize_of_nat(x_29); +lean_dec(x_29); +x_39 = 1; +x_40 = lean_usize_sub(x_38, x_39); +x_41 = lean_usize_land(x_37, x_40); +x_42 = lean_array_uget(x_27, x_41); lean_dec(x_27); -x_37 = 1; -x_38 = lean_usize_sub(x_36, x_37); -x_39 = lean_usize_land(x_35, x_38); -x_40 = lean_array_uget(x_25, x_39); -lean_dec(x_25); -x_41 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__7(x_1, x_40); -lean_dec(x_40); -if (x_41 == 0) +x_43 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__7(x_1, x_42); +lean_dec(x_42); +if (x_43 == 0) { -lean_object* x_42; lean_object* x_43; -lean_free_object(x_23); -x_42 = lean_box(0); -x_43 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_42, x_20, x_21, x_22); +lean_object* x_44; lean_object* x_45; +lean_free_object(x_25); +x_44 = lean_box(0); +x_45 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20, x_44, x_22, x_23, x_24); lean_dec(x_6); -return x_43; +return x_45; } else { -lean_object* x_44; lean_object* x_45; lean_object* x_46; -lean_dec(x_21); -lean_dec(x_20); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_11); +lean_object* x_46; lean_object* x_47; lean_object* x_48; +lean_dec(x_23); +lean_dec(x_22); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_13); +lean_dec(x_12); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -17207,57 +19107,58 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_44 = lean_box(x_17); -lean_ctor_set(x_23, 1, x_18); -lean_ctor_set(x_23, 0, x_44); -x_45 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_45, 0, x_23); -x_46 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_46, 0, x_45); -lean_ctor_set(x_46, 1, x_22); -return x_46; +x_46 = lean_box(x_19); +lean_ctor_set(x_25, 1, x_20); +lean_ctor_set(x_25, 0, x_46); +x_47 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_47, 0, x_25); +x_48 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_48, 0, x_47); +lean_ctor_set(x_48, 1, x_24); +return x_48; } } else { -lean_object* x_47; lean_object* x_48; uint64_t x_49; uint64_t x_50; uint64_t x_51; uint64_t x_52; uint64_t x_53; uint64_t x_54; uint64_t x_55; size_t x_56; size_t x_57; size_t x_58; size_t x_59; size_t x_60; lean_object* x_61; uint8_t x_62; -x_47 = lean_ctor_get(x_23, 1); -lean_inc(x_47); -lean_dec(x_23); -x_48 = lean_array_get_size(x_47); -x_49 = l___private_Lean_Syntax_0__String_hashRange____x40_Lean_Syntax___hyg_169_(x_1); -x_50 = 32; -x_51 = lean_uint64_shift_right(x_49, x_50); -x_52 = lean_uint64_xor(x_49, x_51); -x_53 = 16; -x_54 = lean_uint64_shift_right(x_52, x_53); -x_55 = lean_uint64_xor(x_52, x_54); -x_56 = lean_uint64_to_usize(x_55); -x_57 = lean_usize_of_nat(x_48); -lean_dec(x_48); -x_58 = 1; -x_59 = lean_usize_sub(x_57, x_58); -x_60 = lean_usize_land(x_56, x_59); -x_61 = lean_array_uget(x_47, x_60); -lean_dec(x_47); -x_62 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__7(x_1, x_61); -lean_dec(x_61); -if (x_62 == 0) +lean_object* x_49; lean_object* x_50; uint64_t x_51; uint64_t x_52; uint64_t x_53; uint64_t x_54; uint64_t x_55; uint64_t x_56; uint64_t x_57; size_t x_58; size_t x_59; size_t x_60; size_t x_61; size_t x_62; lean_object* x_63; uint8_t x_64; +x_49 = lean_ctor_get(x_25, 1); +lean_inc(x_49); +lean_dec(x_25); +x_50 = lean_array_get_size(x_49); +x_51 = l___private_Lean_Syntax_0__String_hashRange____x40_Lean_Syntax___hyg_169_(x_1); +x_52 = 32; +x_53 = lean_uint64_shift_right(x_51, x_52); +x_54 = lean_uint64_xor(x_51, x_53); +x_55 = 16; +x_56 = lean_uint64_shift_right(x_54, x_55); +x_57 = lean_uint64_xor(x_54, x_56); +x_58 = lean_uint64_to_usize(x_57); +x_59 = lean_usize_of_nat(x_50); +lean_dec(x_50); +x_60 = 1; +x_61 = lean_usize_sub(x_59, x_60); +x_62 = lean_usize_land(x_58, x_61); +x_63 = lean_array_uget(x_49, x_62); +lean_dec(x_49); +x_64 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__7(x_1, x_63); +lean_dec(x_63); +if (x_64 == 0) { -lean_object* x_63; lean_object* x_64; -x_63 = lean_box(0); -x_64 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_63, x_20, x_21, x_22); +lean_object* x_65; lean_object* x_66; +x_65 = lean_box(0); +x_66 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20, x_65, x_22, x_23, x_24); lean_dec(x_6); -return x_64; +return x_66; } else { -lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; -lean_dec(x_21); -lean_dec(x_20); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_11); +lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; +lean_dec(x_23); +lean_dec(x_22); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_13); +lean_dec(x_12); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -17265,567 +19166,580 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_65 = lean_box(x_17); -x_66 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_66, 0, x_65); -lean_ctor_set(x_66, 1, x_18); -x_67 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_67, 0, x_66); +x_67 = lean_box(x_19); x_68 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_68, 0, x_67); -lean_ctor_set(x_68, 1, x_22); -return x_68; +lean_ctor_set(x_68, 1, x_20); +x_69 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_69, 0, x_68); +x_70 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_70, 0, x_69); +lean_ctor_set(x_70, 1, x_24); +return x_70; } } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, size_t x_13, size_t x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, size_t x_16, size_t x_17, lean_object* x_18, lean_object* x_19, lean_object* x_20, lean_object* x_21) { _start: { -uint8_t x_19; -x_19 = lean_usize_dec_lt(x_14, x_13); -if (x_19 == 0) +uint8_t x_22; +x_22 = lean_usize_dec_lt(x_17, x_16); +if (x_22 == 0) { -lean_object* x_20; -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_11); -lean_dec(x_10); +lean_object* x_23; +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_9); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_20 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_20, 0, x_15); -lean_ctor_set(x_20, 1, x_18); -return x_20; +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_18); +lean_ctor_set(x_23, 1, x_21); +return x_23; } else { -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; -x_21 = lean_array_uget(x_12, x_14); -x_22 = lean_ctor_get(x_21, 1); -lean_inc(x_22); -x_23 = lean_ctor_get(x_21, 0); -lean_inc(x_23); -lean_dec(x_21); -x_24 = lean_ctor_get(x_22, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_22, 1); +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; +x_24 = lean_array_uget(x_15, x_17); +x_25 = lean_ctor_get(x_24, 1); lean_inc(x_25); -x_26 = lean_ctor_get(x_22, 2); +x_26 = lean_ctor_get(x_24, 0); lean_inc(x_26); -x_27 = lean_ctor_get(x_22, 3); +lean_dec(x_24); +x_27 = lean_ctor_get(x_25, 0); lean_inc(x_27); -lean_dec(x_22); -x_28 = !lean_is_exclusive(x_15); -if (x_28 == 0) -{ -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; -x_29 = lean_ctor_get(x_15, 0); -x_30 = lean_ctor_get(x_15, 1); -x_31 = lean_st_ref_get(x_10, x_18); -x_32 = lean_ctor_get(x_31, 0); -lean_inc(x_32); -x_33 = lean_ctor_get(x_31, 1); -lean_inc(x_33); -lean_dec(x_31); -x_34 = lean_array_get_size(x_27); -x_35 = lean_unsigned_to_nat(0u); -x_36 = lean_nat_dec_lt(x_35, x_34); -if (x_36 == 0) +x_28 = lean_ctor_get(x_25, 1); +lean_inc(x_28); +x_29 = lean_ctor_get(x_25, 2); +lean_inc(x_29); +x_30 = lean_ctor_get(x_25, 3); +lean_inc(x_30); +lean_dec(x_25); +x_31 = !lean_is_exclusive(x_18); +if (x_31 == 0) { -lean_object* x_37; uint8_t x_38; lean_object* x_39; +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; +x_32 = lean_ctor_get(x_18, 0); +x_33 = lean_ctor_get(x_18, 1); +x_34 = lean_st_ref_get(x_13, x_21); +x_35 = lean_ctor_get(x_34, 0); +lean_inc(x_35); +x_36 = lean_ctor_get(x_34, 1); +lean_inc(x_36); lean_dec(x_34); +x_37 = lean_array_get_size(x_30); +x_38 = lean_unsigned_to_nat(0u); +x_39 = lean_nat_dec_lt(x_38, x_37); +if (x_39 == 0) +{ +lean_object* x_40; uint8_t x_41; lean_object* x_42; +lean_dec(x_37); +lean_dec(x_35); +lean_free_object(x_18); +x_40 = lean_box(0); +x_41 = lean_unbox(x_32); lean_dec(x_32); -lean_free_object(x_15); -x_37 = lean_box(0); -x_38 = lean_unbox(x_29); -lean_dec(x_29); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_11); -lean_inc(x_6); -lean_inc(x_10); +lean_inc(x_20); +lean_inc(x_19); +lean_inc(x_14); lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_13); +lean_inc(x_9); lean_inc(x_5); lean_inc(x_1); -x_39 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__6(x_23, x_1, x_25, x_24, x_5, x_7, x_10, x_27, x_8, x_9, x_6, x_4, x_3, x_11, x_26, x_2, x_38, x_30, x_37, x_16, x_17, x_33); -lean_dec(x_27); -if (lean_obj_tag(x_39) == 0) +x_42 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__6(x_26, x_1, x_28, x_27, x_5, x_9, x_13, x_30, x_11, x_12, x_10, x_6, x_7, x_4, x_3, x_14, x_29, x_2, x_41, x_33, x_40, x_19, x_20, x_36); +lean_dec(x_30); +if (lean_obj_tag(x_42) == 0) { -lean_object* x_40; -x_40 = lean_ctor_get(x_39, 0); -lean_inc(x_40); -if (lean_obj_tag(x_40) == 0) +lean_object* x_43; +x_43 = lean_ctor_get(x_42, 0); +lean_inc(x_43); +if (lean_obj_tag(x_43) == 0) { -uint8_t x_41; -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_11); -lean_dec(x_10); +uint8_t x_44; +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_9); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_41 = !lean_is_exclusive(x_39); -if (x_41 == 0) +x_44 = !lean_is_exclusive(x_42); +if (x_44 == 0) { -lean_object* x_42; lean_object* x_43; -x_42 = lean_ctor_get(x_39, 0); -lean_dec(x_42); -x_43 = lean_ctor_get(x_40, 0); -lean_inc(x_43); -lean_dec(x_40); -lean_ctor_set(x_39, 0, x_43); -return x_39; +lean_object* x_45; lean_object* x_46; +x_45 = lean_ctor_get(x_42, 0); +lean_dec(x_45); +x_46 = lean_ctor_get(x_43, 0); +lean_inc(x_46); +lean_dec(x_43); +lean_ctor_set(x_42, 0, x_46); +return x_42; } else { -lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_44 = lean_ctor_get(x_39, 1); -lean_inc(x_44); -lean_dec(x_39); -x_45 = lean_ctor_get(x_40, 0); -lean_inc(x_45); -lean_dec(x_40); -x_46 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_46, 0, x_45); -lean_ctor_set(x_46, 1, x_44); -return x_46; +lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_47 = lean_ctor_get(x_42, 1); +lean_inc(x_47); +lean_dec(x_42); +x_48 = lean_ctor_get(x_43, 0); +lean_inc(x_48); +lean_dec(x_43); +x_49 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_49, 0, x_48); +lean_ctor_set(x_49, 1, x_47); +return x_49; } } else { -lean_object* x_47; lean_object* x_48; size_t x_49; size_t x_50; -x_47 = lean_ctor_get(x_39, 1); -lean_inc(x_47); -lean_dec(x_39); -x_48 = lean_ctor_get(x_40, 0); -lean_inc(x_48); -lean_dec(x_40); -x_49 = 1; -x_50 = lean_usize_add(x_14, x_49); -x_14 = x_50; -x_15 = x_48; -x_18 = x_47; +lean_object* x_50; lean_object* x_51; size_t x_52; size_t x_53; +x_50 = lean_ctor_get(x_42, 1); +lean_inc(x_50); +lean_dec(x_42); +x_51 = lean_ctor_get(x_43, 0); +lean_inc(x_51); +lean_dec(x_43); +x_52 = 1; +x_53 = lean_usize_add(x_17, x_52); +x_17 = x_53; +x_18 = x_51; +x_21 = x_50; goto _start; } } else { -uint8_t x_52; -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_11); -lean_dec(x_10); +uint8_t x_55; +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_9); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_52 = !lean_is_exclusive(x_39); -if (x_52 == 0) +x_55 = !lean_is_exclusive(x_42); +if (x_55 == 0) { -return x_39; +return x_42; } else { -lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_53 = lean_ctor_get(x_39, 0); -x_54 = lean_ctor_get(x_39, 1); -lean_inc(x_54); -lean_inc(x_53); -lean_dec(x_39); -x_55 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_55, 0, x_53); -lean_ctor_set(x_55, 1, x_54); -return x_55; +lean_object* x_56; lean_object* x_57; lean_object* x_58; +x_56 = lean_ctor_get(x_42, 0); +x_57 = lean_ctor_get(x_42, 1); +lean_inc(x_57); +lean_inc(x_56); +lean_dec(x_42); +x_58 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_58, 0, x_56); +lean_ctor_set(x_58, 1, x_57); +return x_58; } } } else { -size_t x_56; size_t x_57; uint8_t x_58; -x_56 = 0; -x_57 = lean_usize_of_nat(x_34); -lean_dec(x_34); -x_58 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__18(x_8, x_9, x_32, x_27, x_56, x_57); -lean_dec(x_32); -if (x_58 == 0) +size_t x_59; size_t x_60; uint8_t x_61; +x_59 = 0; +x_60 = lean_usize_of_nat(x_37); +lean_dec(x_37); +x_61 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__24(x_11, x_12, x_35, x_30, x_59, x_60); +lean_dec(x_35); +if (x_61 == 0) { -lean_object* x_59; uint8_t x_60; lean_object* x_61; -lean_free_object(x_15); -x_59 = lean_box(0); -x_60 = lean_unbox(x_29); -lean_dec(x_29); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_11); -lean_inc(x_6); -lean_inc(x_10); +lean_object* x_62; uint8_t x_63; lean_object* x_64; +lean_free_object(x_18); +x_62 = lean_box(0); +x_63 = lean_unbox(x_32); +lean_dec(x_32); +lean_inc(x_20); +lean_inc(x_19); +lean_inc(x_14); lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_13); +lean_inc(x_9); lean_inc(x_5); lean_inc(x_1); -x_61 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__6(x_23, x_1, x_25, x_24, x_5, x_7, x_10, x_27, x_8, x_9, x_6, x_4, x_3, x_11, x_26, x_2, x_60, x_30, x_59, x_16, x_17, x_33); -lean_dec(x_27); -if (lean_obj_tag(x_61) == 0) +x_64 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__6(x_26, x_1, x_28, x_27, x_5, x_9, x_13, x_30, x_11, x_12, x_10, x_6, x_7, x_4, x_3, x_14, x_29, x_2, x_63, x_33, x_62, x_19, x_20, x_36); +lean_dec(x_30); +if (lean_obj_tag(x_64) == 0) { -lean_object* x_62; -x_62 = lean_ctor_get(x_61, 0); -lean_inc(x_62); -if (lean_obj_tag(x_62) == 0) +lean_object* x_65; +x_65 = lean_ctor_get(x_64, 0); +lean_inc(x_65); +if (lean_obj_tag(x_65) == 0) { -uint8_t x_63; -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_11); -lean_dec(x_10); +uint8_t x_66; +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_9); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_63 = !lean_is_exclusive(x_61); -if (x_63 == 0) +x_66 = !lean_is_exclusive(x_64); +if (x_66 == 0) { -lean_object* x_64; lean_object* x_65; -x_64 = lean_ctor_get(x_61, 0); -lean_dec(x_64); -x_65 = lean_ctor_get(x_62, 0); -lean_inc(x_65); -lean_dec(x_62); -lean_ctor_set(x_61, 0, x_65); -return x_61; +lean_object* x_67; lean_object* x_68; +x_67 = lean_ctor_get(x_64, 0); +lean_dec(x_67); +x_68 = lean_ctor_get(x_65, 0); +lean_inc(x_68); +lean_dec(x_65); +lean_ctor_set(x_64, 0, x_68); +return x_64; } else { -lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_66 = lean_ctor_get(x_61, 1); -lean_inc(x_66); -lean_dec(x_61); -x_67 = lean_ctor_get(x_62, 0); -lean_inc(x_67); -lean_dec(x_62); -x_68 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_68, 0, x_67); -lean_ctor_set(x_68, 1, x_66); -return x_68; +lean_object* x_69; lean_object* x_70; lean_object* x_71; +x_69 = lean_ctor_get(x_64, 1); +lean_inc(x_69); +lean_dec(x_64); +x_70 = lean_ctor_get(x_65, 0); +lean_inc(x_70); +lean_dec(x_65); +x_71 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_71, 0, x_70); +lean_ctor_set(x_71, 1, x_69); +return x_71; } } else { -lean_object* x_69; lean_object* x_70; size_t x_71; size_t x_72; -x_69 = lean_ctor_get(x_61, 1); -lean_inc(x_69); -lean_dec(x_61); -x_70 = lean_ctor_get(x_62, 0); -lean_inc(x_70); -lean_dec(x_62); -x_71 = 1; -x_72 = lean_usize_add(x_14, x_71); -x_14 = x_72; -x_15 = x_70; -x_18 = x_69; +lean_object* x_72; lean_object* x_73; size_t x_74; size_t x_75; +x_72 = lean_ctor_get(x_64, 1); +lean_inc(x_72); +lean_dec(x_64); +x_73 = lean_ctor_get(x_65, 0); +lean_inc(x_73); +lean_dec(x_65); +x_74 = 1; +x_75 = lean_usize_add(x_17, x_74); +x_17 = x_75; +x_18 = x_73; +x_21 = x_72; goto _start; } } else { -uint8_t x_74; -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_11); -lean_dec(x_10); +uint8_t x_77; +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_9); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_74 = !lean_is_exclusive(x_61); -if (x_74 == 0) +x_77 = !lean_is_exclusive(x_64); +if (x_77 == 0) { -return x_61; +return x_64; } else { -lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_75 = lean_ctor_get(x_61, 0); -x_76 = lean_ctor_get(x_61, 1); -lean_inc(x_76); -lean_inc(x_75); -lean_dec(x_61); -x_77 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_77, 0, x_75); -lean_ctor_set(x_77, 1, x_76); -return x_77; +lean_object* x_78; lean_object* x_79; lean_object* x_80; +x_78 = lean_ctor_get(x_64, 0); +x_79 = lean_ctor_get(x_64, 1); +lean_inc(x_79); +lean_inc(x_78); +lean_dec(x_64); +x_80 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_80, 0, x_78); +lean_ctor_set(x_80, 1, x_79); +return x_80; } } } else { -size_t x_78; size_t x_79; +size_t x_81; size_t x_82; +lean_dec(x_30); +lean_dec(x_29); +lean_dec(x_28); lean_dec(x_27); lean_dec(x_26); -lean_dec(x_25); -lean_dec(x_24); -lean_dec(x_23); -x_78 = 1; -x_79 = lean_usize_add(x_14, x_78); -x_14 = x_79; -x_18 = x_33; +x_81 = 1; +x_82 = lean_usize_add(x_17, x_81); +x_17 = x_82; +x_21 = x_36; goto _start; } } } else { -lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; uint8_t x_88; -x_81 = lean_ctor_get(x_15, 0); -x_82 = lean_ctor_get(x_15, 1); -lean_inc(x_82); -lean_inc(x_81); -lean_dec(x_15); -x_83 = lean_st_ref_get(x_10, x_18); -x_84 = lean_ctor_get(x_83, 0); -lean_inc(x_84); -x_85 = lean_ctor_get(x_83, 1); +lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; uint8_t x_91; +x_84 = lean_ctor_get(x_18, 0); +x_85 = lean_ctor_get(x_18, 1); lean_inc(x_85); -lean_dec(x_83); -x_86 = lean_array_get_size(x_27); -x_87 = lean_unsigned_to_nat(0u); -x_88 = lean_nat_dec_lt(x_87, x_86); -if (x_88 == 0) -{ -lean_object* x_89; uint8_t x_90; lean_object* x_91; +lean_inc(x_84); +lean_dec(x_18); +x_86 = lean_st_ref_get(x_13, x_21); +x_87 = lean_ctor_get(x_86, 0); +lean_inc(x_87); +x_88 = lean_ctor_get(x_86, 1); +lean_inc(x_88); lean_dec(x_86); +x_89 = lean_array_get_size(x_30); +x_90 = lean_unsigned_to_nat(0u); +x_91 = lean_nat_dec_lt(x_90, x_89); +if (x_91 == 0) +{ +lean_object* x_92; uint8_t x_93; lean_object* x_94; +lean_dec(x_89); +lean_dec(x_87); +x_92 = lean_box(0); +x_93 = lean_unbox(x_84); lean_dec(x_84); -x_89 = lean_box(0); -x_90 = lean_unbox(x_81); -lean_dec(x_81); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_11); -lean_inc(x_6); -lean_inc(x_10); +lean_inc(x_20); +lean_inc(x_19); +lean_inc(x_14); lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_13); +lean_inc(x_9); lean_inc(x_5); lean_inc(x_1); -x_91 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__6(x_23, x_1, x_25, x_24, x_5, x_7, x_10, x_27, x_8, x_9, x_6, x_4, x_3, x_11, x_26, x_2, x_90, x_82, x_89, x_16, x_17, x_85); -lean_dec(x_27); -if (lean_obj_tag(x_91) == 0) +x_94 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__6(x_26, x_1, x_28, x_27, x_5, x_9, x_13, x_30, x_11, x_12, x_10, x_6, x_7, x_4, x_3, x_14, x_29, x_2, x_93, x_85, x_92, x_19, x_20, x_88); +lean_dec(x_30); +if (lean_obj_tag(x_94) == 0) { -lean_object* x_92; -x_92 = lean_ctor_get(x_91, 0); -lean_inc(x_92); -if (lean_obj_tag(x_92) == 0) +lean_object* x_95; +x_95 = lean_ctor_get(x_94, 0); +lean_inc(x_95); +if (lean_obj_tag(x_95) == 0) { -lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_11); -lean_dec(x_10); +lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_9); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_93 = lean_ctor_get(x_91, 1); -lean_inc(x_93); -if (lean_is_exclusive(x_91)) { - lean_ctor_release(x_91, 0); - lean_ctor_release(x_91, 1); - x_94 = x_91; +x_96 = lean_ctor_get(x_94, 1); +lean_inc(x_96); +if (lean_is_exclusive(x_94)) { + lean_ctor_release(x_94, 0); + lean_ctor_release(x_94, 1); + x_97 = x_94; } else { - lean_dec_ref(x_91); - x_94 = lean_box(0); + lean_dec_ref(x_94); + x_97 = lean_box(0); } -x_95 = lean_ctor_get(x_92, 0); -lean_inc(x_95); -lean_dec(x_92); -if (lean_is_scalar(x_94)) { - x_96 = lean_alloc_ctor(0, 2, 0); +x_98 = lean_ctor_get(x_95, 0); +lean_inc(x_98); +lean_dec(x_95); +if (lean_is_scalar(x_97)) { + x_99 = lean_alloc_ctor(0, 2, 0); } else { - x_96 = x_94; + x_99 = x_97; } -lean_ctor_set(x_96, 0, x_95); -lean_ctor_set(x_96, 1, x_93); -return x_96; +lean_ctor_set(x_99, 0, x_98); +lean_ctor_set(x_99, 1, x_96); +return x_99; } else { -lean_object* x_97; lean_object* x_98; size_t x_99; size_t x_100; -x_97 = lean_ctor_get(x_91, 1); -lean_inc(x_97); -lean_dec(x_91); -x_98 = lean_ctor_get(x_92, 0); -lean_inc(x_98); -lean_dec(x_92); -x_99 = 1; -x_100 = lean_usize_add(x_14, x_99); -x_14 = x_100; -x_15 = x_98; -x_18 = x_97; +lean_object* x_100; lean_object* x_101; size_t x_102; size_t x_103; +x_100 = lean_ctor_get(x_94, 1); +lean_inc(x_100); +lean_dec(x_94); +x_101 = lean_ctor_get(x_95, 0); +lean_inc(x_101); +lean_dec(x_95); +x_102 = 1; +x_103 = lean_usize_add(x_17, x_102); +x_17 = x_103; +x_18 = x_101; +x_21 = x_100; goto _start; } } else { -lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_11); -lean_dec(x_10); +lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_9); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_102 = lean_ctor_get(x_91, 0); -lean_inc(x_102); -x_103 = lean_ctor_get(x_91, 1); -lean_inc(x_103); -if (lean_is_exclusive(x_91)) { - lean_ctor_release(x_91, 0); - lean_ctor_release(x_91, 1); - x_104 = x_91; +x_105 = lean_ctor_get(x_94, 0); +lean_inc(x_105); +x_106 = lean_ctor_get(x_94, 1); +lean_inc(x_106); +if (lean_is_exclusive(x_94)) { + lean_ctor_release(x_94, 0); + lean_ctor_release(x_94, 1); + x_107 = x_94; } else { - lean_dec_ref(x_91); - x_104 = lean_box(0); + lean_dec_ref(x_94); + x_107 = lean_box(0); } -if (lean_is_scalar(x_104)) { - x_105 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_107)) { + x_108 = lean_alloc_ctor(1, 2, 0); } else { - x_105 = x_104; + x_108 = x_107; } -lean_ctor_set(x_105, 0, x_102); -lean_ctor_set(x_105, 1, x_103); -return x_105; +lean_ctor_set(x_108, 0, x_105); +lean_ctor_set(x_108, 1, x_106); +return x_108; } } else { -size_t x_106; size_t x_107; uint8_t x_108; -x_106 = 0; -x_107 = lean_usize_of_nat(x_86); -lean_dec(x_86); -x_108 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__18(x_8, x_9, x_84, x_27, x_106, x_107); -lean_dec(x_84); -if (x_108 == 0) +size_t x_109; size_t x_110; uint8_t x_111; +x_109 = 0; +x_110 = lean_usize_of_nat(x_89); +lean_dec(x_89); +x_111 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__24(x_11, x_12, x_87, x_30, x_109, x_110); +lean_dec(x_87); +if (x_111 == 0) { -lean_object* x_109; uint8_t x_110; lean_object* x_111; -x_109 = lean_box(0); -x_110 = lean_unbox(x_81); -lean_dec(x_81); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_11); -lean_inc(x_6); -lean_inc(x_10); +lean_object* x_112; uint8_t x_113; lean_object* x_114; +x_112 = lean_box(0); +x_113 = lean_unbox(x_84); +lean_dec(x_84); +lean_inc(x_20); +lean_inc(x_19); +lean_inc(x_14); lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_13); +lean_inc(x_9); lean_inc(x_5); lean_inc(x_1); -x_111 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__6(x_23, x_1, x_25, x_24, x_5, x_7, x_10, x_27, x_8, x_9, x_6, x_4, x_3, x_11, x_26, x_2, x_110, x_82, x_109, x_16, x_17, x_85); -lean_dec(x_27); -if (lean_obj_tag(x_111) == 0) +x_114 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__6(x_26, x_1, x_28, x_27, x_5, x_9, x_13, x_30, x_11, x_12, x_10, x_6, x_7, x_4, x_3, x_14, x_29, x_2, x_113, x_85, x_112, x_19, x_20, x_88); +lean_dec(x_30); +if (lean_obj_tag(x_114) == 0) { -lean_object* x_112; -x_112 = lean_ctor_get(x_111, 0); -lean_inc(x_112); -if (lean_obj_tag(x_112) == 0) +lean_object* x_115; +x_115 = lean_ctor_get(x_114, 0); +lean_inc(x_115); +if (lean_obj_tag(x_115) == 0) { -lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_11); -lean_dec(x_10); +lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_9); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_113 = lean_ctor_get(x_111, 1); -lean_inc(x_113); -if (lean_is_exclusive(x_111)) { - lean_ctor_release(x_111, 0); - lean_ctor_release(x_111, 1); - x_114 = x_111; +x_116 = lean_ctor_get(x_114, 1); +lean_inc(x_116); +if (lean_is_exclusive(x_114)) { + lean_ctor_release(x_114, 0); + lean_ctor_release(x_114, 1); + x_117 = x_114; } else { - lean_dec_ref(x_111); - x_114 = lean_box(0); + lean_dec_ref(x_114); + x_117 = lean_box(0); } -x_115 = lean_ctor_get(x_112, 0); -lean_inc(x_115); -lean_dec(x_112); -if (lean_is_scalar(x_114)) { - x_116 = lean_alloc_ctor(0, 2, 0); +x_118 = lean_ctor_get(x_115, 0); +lean_inc(x_118); +lean_dec(x_115); +if (lean_is_scalar(x_117)) { + x_119 = lean_alloc_ctor(0, 2, 0); } else { - x_116 = x_114; + x_119 = x_117; } -lean_ctor_set(x_116, 0, x_115); -lean_ctor_set(x_116, 1, x_113); -return x_116; +lean_ctor_set(x_119, 0, x_118); +lean_ctor_set(x_119, 1, x_116); +return x_119; } else { -lean_object* x_117; lean_object* x_118; size_t x_119; size_t x_120; -x_117 = lean_ctor_get(x_111, 1); -lean_inc(x_117); -lean_dec(x_111); -x_118 = lean_ctor_get(x_112, 0); -lean_inc(x_118); -lean_dec(x_112); -x_119 = 1; -x_120 = lean_usize_add(x_14, x_119); -x_14 = x_120; -x_15 = x_118; -x_18 = x_117; +lean_object* x_120; lean_object* x_121; size_t x_122; size_t x_123; +x_120 = lean_ctor_get(x_114, 1); +lean_inc(x_120); +lean_dec(x_114); +x_121 = lean_ctor_get(x_115, 0); +lean_inc(x_121); +lean_dec(x_115); +x_122 = 1; +x_123 = lean_usize_add(x_17, x_122); +x_17 = x_123; +x_18 = x_121; +x_21 = x_120; goto _start; } } else { -lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_11); -lean_dec(x_10); +lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_9); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_122 = lean_ctor_get(x_111, 0); -lean_inc(x_122); -x_123 = lean_ctor_get(x_111, 1); -lean_inc(x_123); -if (lean_is_exclusive(x_111)) { - lean_ctor_release(x_111, 0); - lean_ctor_release(x_111, 1); - x_124 = x_111; +x_125 = lean_ctor_get(x_114, 0); +lean_inc(x_125); +x_126 = lean_ctor_get(x_114, 1); +lean_inc(x_126); +if (lean_is_exclusive(x_114)) { + lean_ctor_release(x_114, 0); + lean_ctor_release(x_114, 1); + x_127 = x_114; } else { - lean_dec_ref(x_111); - x_124 = lean_box(0); + lean_dec_ref(x_114); + x_127 = lean_box(0); } -if (lean_is_scalar(x_124)) { - x_125 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_127)) { + x_128 = lean_alloc_ctor(1, 2, 0); } else { - x_125 = x_124; + x_128 = x_127; } -lean_ctor_set(x_125, 0, x_122); -lean_ctor_set(x_125, 1, x_123); -return x_125; +lean_ctor_set(x_128, 0, x_125); +lean_ctor_set(x_128, 1, x_126); +return x_128; } } else { -lean_object* x_126; size_t x_127; size_t x_128; +lean_object* x_129; size_t x_130; size_t x_131; +lean_dec(x_30); +lean_dec(x_29); +lean_dec(x_28); lean_dec(x_27); lean_dec(x_26); -lean_dec(x_25); -lean_dec(x_24); -lean_dec(x_23); -x_126 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_126, 0, x_81); -lean_ctor_set(x_126, 1, x_82); -x_127 = 1; -x_128 = lean_usize_add(x_14, x_127); -x_14 = x_128; -x_15 = x_126; -x_18 = x_85; +x_129 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_129, 0, x_84); +lean_ctor_set(x_129, 1, x_85); +x_130 = 1; +x_131 = lean_usize_add(x_17, x_130); +x_17 = x_131; +x_18 = x_129; +x_21 = x_88; goto _start; } } @@ -17833,7 +19747,7 @@ goto _start; } } } -static lean_object* _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__1() { +static lean_object* _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__1() { _start: { lean_object* x_1; @@ -17841,7 +19755,7 @@ x_1 = lean_mk_string_unchecked("Init.Data.Option.BasicAux", 25, 25); return x_1; } } -static lean_object* _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__2() { +static lean_object* _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__2() { _start: { lean_object* x_1; @@ -17849,7 +19763,7 @@ x_1 = lean_mk_string_unchecked("Option.get!", 11, 11); return x_1; } } -static lean_object* _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__3() { +static lean_object* _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__3() { _start: { lean_object* x_1; @@ -17857,20 +19771,20 @@ x_1 = lean_mk_string_unchecked("value is none", 13, 13); return x_1; } } -static lean_object* _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__4() { +static lean_object* _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__1; -x_2 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__2; +x_1 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__1; +x_2 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__2; x_3 = lean_unsigned_to_nat(16u); x_4 = lean_unsigned_to_nat(14u); -x_5 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__3; +x_5 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; } } -LEAN_EXPORT uint8_t l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; @@ -17882,7 +19796,7 @@ x_7 = l_Lean_Syntax_getPos_x3f(x_6, x_4); if (lean_obj_tag(x_5) == 0) { lean_object* x_8; lean_object* x_9; -x_8 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__4; +x_8 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__4; x_9 = l_panic___at_Lean_Parser_ParserState_mkUnexpectedTokenErrors___spec__1(x_8); if (lean_obj_tag(x_7) == 0) { @@ -17913,7 +19827,7 @@ lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; x_14 = lean_ctor_get(x_5, 0); lean_inc(x_14); lean_dec(x_5); -x_15 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__4; +x_15 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__4; x_16 = l_panic___at_Lean_Parser_ParserState_mkUnexpectedTokenErrors___spec__1(x_15); x_17 = lean_nat_dec_lt(x_14, x_16); lean_dec(x_16); @@ -17937,15 +19851,15 @@ return x_20; } } } -static lean_object* _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___closed__1() { +static lean_object* _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___boxed), 2, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -17958,7 +19872,7 @@ return x_1; else { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; -x_5 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___closed__1; +x_5 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___closed__1; lean_inc(x_2); x_6 = l_Array_qpartition___rarg(x_1, x_5, x_2, x_3); x_7 = lean_ctor_get(x_6, 0); @@ -17970,7 +19884,7 @@ x_9 = lean_nat_dec_le(x_3, x_7); if (x_9 == 0) { lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_10 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20(x_8, x_2, x_7); +x_10 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26(x_8, x_2, x_7); x_11 = lean_unsigned_to_nat(1u); x_12 = lean_nat_add(x_7, x_11); lean_dec(x_7); @@ -17987,7 +19901,7 @@ return x_8; } } } -static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__1() { +static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__1() { _start: { lean_object* x_1; @@ -17995,16 +19909,16 @@ x_1 = lean_mk_string_unchecked("note: this linter can be disabled with `set_opti return x_1; } } -static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__2() { +static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__1; +x_1 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__3() { +static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__3() { _start: { lean_object* x_1; @@ -18012,16 +19926,16 @@ x_1 = lean_mk_string_unchecked(" false`", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__4() { +static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__3; +x_1 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__3; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__5() { +static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__5() { _start: { lean_object* x_1; lean_object* x_2; @@ -18030,7 +19944,7 @@ x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__6() { +static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__6() { _start: { lean_object* x_1; @@ -18038,16 +19952,16 @@ x_1 = lean_mk_string_unchecked("\n", 1, 1); return x_1; } } -static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__7() { +static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__7() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__6; +x_1 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__6; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { uint8_t x_7; @@ -18060,19 +19974,19 @@ x_9 = lean_ctor_get(x_1, 1); lean_dec(x_9); lean_inc(x_8); x_10 = l_Lean_MessageData_ofName(x_8); -x_11 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__2; +x_11 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__2; lean_ctor_set_tag(x_1, 7); lean_ctor_set(x_1, 1, x_10); lean_ctor_set(x_1, 0, x_11); -x_12 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__4; +x_12 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__4; x_13 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_13, 0, x_1); lean_ctor_set(x_13, 1, x_12); -x_14 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__5; +x_14 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__5; x_15 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_15, 0, x_14); lean_ctor_set(x_15, 1, x_3); -x_16 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__7; +x_16 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__7; x_17 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_17, 0, x_15); lean_ctor_set(x_17, 1, x_16); @@ -18097,19 +20011,19 @@ lean_inc(x_23); lean_dec(x_1); lean_inc(x_23); x_24 = l_Lean_MessageData_ofName(x_23); -x_25 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__2; +x_25 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__2; x_26 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_26, 0, x_25); lean_ctor_set(x_26, 1, x_24); -x_27 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__4; +x_27 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__4; x_28 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_28, 0, x_26); lean_ctor_set(x_28, 1, x_27); -x_29 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__5; +x_29 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__5; x_30 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_30, 0, x_29); lean_ctor_set(x_30, 1, x_3); -x_31 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__7; +x_31 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__7; x_32 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_32, 0, x_30); lean_ctor_set(x_32, 1, x_31); @@ -18128,7 +20042,7 @@ return x_37; } } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__1() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__1() { _start: { lean_object* x_1; @@ -18136,16 +20050,16 @@ x_1 = lean_mk_string_unchecked("unused variable `", 17, 17); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__2() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__1; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__3() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__3() { _start: { lean_object* x_1; @@ -18153,16 +20067,16 @@ x_1 = lean_mk_string_unchecked("`", 1, 1); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__4() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__3; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__3; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { uint8_t x_8; @@ -18188,17 +20102,17 @@ lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean x_12 = lean_ctor_get(x_10, 0); x_13 = lean_ctor_get(x_10, 1); x_14 = l_Lean_MessageData_ofName(x_13); -x_15 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__2; +x_15 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__2; lean_ctor_set_tag(x_10, 7); lean_ctor_set(x_10, 1, x_14); lean_ctor_set(x_10, 0, x_15); -x_16 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__4; +x_16 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__4; x_17 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_17, 0, x_10); lean_ctor_set(x_17, 1, x_16); x_18 = l_Lean_Linter_getLinterUnusedVariables___closed__1; lean_inc(x_5); -x_19 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21(x_18, x_12, x_17, x_5, x_6, x_7); +x_19 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27(x_18, x_12, x_17, x_5, x_6, x_7); lean_dec(x_12); x_20 = lean_ctor_get(x_19, 1); lean_inc(x_20); @@ -18220,17 +20134,17 @@ lean_inc(x_26); lean_inc(x_25); lean_dec(x_10); x_27 = l_Lean_MessageData_ofName(x_26); -x_28 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__2; +x_28 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__2; x_29 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_29, 0, x_28); lean_ctor_set(x_29, 1, x_27); -x_30 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__4; +x_30 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__4; x_31 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_31, 0, x_29); lean_ctor_set(x_31, 1, x_30); x_32 = l_Lean_Linter_getLinterUnusedVariables___closed__1; lean_inc(x_5); -x_33 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21(x_32, x_25, x_31, x_5, x_6, x_7); +x_33 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27(x_32, x_25, x_31, x_5, x_6, x_7); lean_dec(x_25); x_34 = lean_ctor_get(x_33, 1); lean_inc(x_34); @@ -18246,7 +20160,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__23(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__29(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { uint8_t x_5; @@ -18255,7 +20169,7 @@ if (x_5 == 0) { lean_object* x_6; lean_object* x_7; size_t x_8; size_t x_9; x_6 = lean_array_uget(x_1, x_2); -x_7 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__3(x_4, x_6); +x_7 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__4(x_4, x_6); lean_dec(x_6); x_8 = 1; x_9 = lean_usize_add(x_2, x_8); @@ -18269,7 +20183,7 @@ return x_4; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__24(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__30(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { uint8_t x_5; @@ -18291,7 +20205,7 @@ return x_4; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__31(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6) { _start: { uint8_t x_7; @@ -18315,7 +20229,7 @@ return x_6; } } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__32(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { uint8_t x_7; @@ -18447,9 +20361,8 @@ if (x_18 == 0) { lean_dec(x_16); lean_dec(x_15); -lean_dec(x_9); -lean_inc(x_8); -x_20 = x_8; +lean_inc(x_9); +x_20 = x_9; goto block_110; } else @@ -18460,9 +20373,8 @@ if (x_111 == 0) { lean_dec(x_16); lean_dec(x_15); -lean_dec(x_9); -lean_inc(x_8); -x_20 = x_8; +lean_inc(x_9); +x_20 = x_9; goto block_110; } else @@ -18471,8 +20383,9 @@ size_t x_112; size_t x_113; lean_object* x_114; x_112 = 0; x_113 = lean_usize_of_nat(x_16); lean_dec(x_16); +lean_inc(x_9); lean_inc(x_8); -x_114 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25(x_9, x_1, x_15, x_112, x_113, x_8); +x_114 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__31(x_8, x_1, x_15, x_112, x_113, x_9); lean_dec(x_15); x_20 = x_114; goto block_110; @@ -18525,7 +20438,7 @@ size_t x_104; size_t x_105; lean_object* x_106; lean_object* x_107; lean_object* x_104 = 0; x_105 = lean_usize_of_nat(x_22); lean_dec(x_22); -x_106 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__24(x_21, x_104, x_105, x_19); +x_106 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__30(x_21, x_104, x_105, x_19); lean_dec(x_21); x_107 = lean_st_mk_ref(x_106, x_13); x_108 = lean_ctor_get(x_107, 0); @@ -18584,7 +20497,7 @@ else size_t x_60; lean_object* x_61; x_60 = lean_usize_of_nat(x_32); lean_dec(x_32); -x_61 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__23(x_31, x_36, x_60, x_2); +x_61 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__29(x_31, x_36, x_60, x_2); lean_dec(x_31); x_37 = x_61; goto block_58; @@ -18596,9 +20509,11 @@ size_t x_38; lean_object* x_39; x_38 = lean_array_size(x_37); lean_inc(x_12); lean_inc(x_11); -x_39 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19(x_3, x_4, x_5, x_6, x_7, x_8, x_1, x_20, x_20, x_24, x_28, x_37, x_38, x_36, x_26, x_11, x_12, x_29); +lean_inc(x_9); +x_39 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_9, x_1, x_20, x_20, x_20, x_24, x_28, x_37, x_38, x_36, x_26, x_11, x_12, x_29); lean_dec(x_37); lean_dec(x_20); +lean_dec(x_9); if (lean_obj_tag(x_39) == 0) { lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; size_t x_47; lean_object* x_48; lean_object* x_49; uint8_t x_50; @@ -18614,11 +20529,11 @@ x_43 = lean_array_get_size(x_42); x_44 = lean_unsigned_to_nat(1u); x_45 = lean_nat_sub(x_43, x_44); lean_dec(x_43); -x_46 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20(x_42, x_17, x_45); +x_46 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26(x_42, x_17, x_45); lean_dec(x_45); x_47 = lean_array_size(x_46); x_48 = lean_box(0); -x_49 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22(x_46, x_47, x_36, x_48, x_11, x_12, x_41); +x_49 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28(x_46, x_47, x_36, x_48, x_11, x_12, x_41); lean_dec(x_12); lean_dec(x_46); x_50 = !lean_is_exclusive(x_49); @@ -18713,7 +20628,7 @@ else size_t x_94; lean_object* x_95; x_94 = lean_usize_of_nat(x_66); lean_dec(x_66); -x_95 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__23(x_65, x_71, x_94, x_2); +x_95 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__29(x_65, x_71, x_94, x_2); lean_dec(x_65); x_72 = x_95; goto block_92; @@ -18725,9 +20640,11 @@ size_t x_73; lean_object* x_74; x_73 = lean_array_size(x_72); lean_inc(x_12); lean_inc(x_11); -x_74 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19(x_3, x_4, x_5, x_6, x_7, x_8, x_1, x_20, x_20, x_24, x_62, x_72, x_73, x_71, x_70, x_11, x_12, x_63); +lean_inc(x_9); +x_74 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_9, x_1, x_20, x_20, x_20, x_24, x_62, x_72, x_73, x_71, x_70, x_11, x_12, x_63); lean_dec(x_72); lean_dec(x_20); +lean_dec(x_9); if (lean_obj_tag(x_74) == 0) { lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; size_t x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; @@ -18743,11 +20660,11 @@ x_78 = lean_array_get_size(x_77); x_79 = lean_unsigned_to_nat(1u); x_80 = lean_nat_sub(x_78, x_79); lean_dec(x_78); -x_81 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20(x_77, x_17, x_80); +x_81 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26(x_77, x_17, x_80); lean_dec(x_80); x_82 = lean_array_size(x_81); x_83 = lean_box(0); -x_84 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22(x_81, x_82, x_71, x_83, x_11, x_12, x_76); +x_84 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28(x_81, x_82, x_71, x_83, x_11, x_12, x_76); lean_dec(x_12); lean_dec(x_81); x_85 = lean_ctor_get(x_84, 1); @@ -18806,7 +20723,7 @@ static lean_object* _init_l_Lean_Linter_UnusedVariables_unusedVariables___elambd { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Linter_UnusedVariables_visitAssignments___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_340____closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379____closed__1; x_3 = lean_alloc_ctor(0, 5, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_1); @@ -18858,11 +20775,11 @@ if (x_25 == 0) { lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_free_object(x_18); -x_26 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_340____closed__1; +x_26 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379____closed__1; x_27 = l_Lean_Linter_UnusedVariables_visitAssignments___closed__1; x_28 = l_Lean_Linter_UnusedVariables_visitAssignments___closed__3; x_29 = lean_box(0); -x_30 = l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___lambda__1(x_20, x_26, x_3, x_1, x_4, x_5, x_27, x_28, x_10, x_29, x_7, x_8, x_21); +x_30 = l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___lambda__1(x_20, x_26, x_3, x_1, x_4, x_5, x_27, x_10, x_28, x_29, x_7, x_8, x_21); return x_30; } else @@ -18896,11 +20813,11 @@ lean_dec(x_35); if (x_37 == 0) { lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_38 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_340____closed__1; +x_38 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379____closed__1; x_39 = l_Lean_Linter_UnusedVariables_visitAssignments___closed__1; x_40 = l_Lean_Linter_UnusedVariables_visitAssignments___closed__3; x_41 = lean_box(0); -x_42 = l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___lambda__1(x_32, x_38, x_3, x_1, x_4, x_5, x_39, x_40, x_10, x_41, x_7, x_8, x_33); +x_42 = l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___lambda__1(x_32, x_38, x_3, x_1, x_4, x_5, x_39, x_10, x_40, x_41, x_7, x_8, x_33); return x_42; } else @@ -19007,11 +20924,11 @@ if (x_69 == 0) { lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_dec(x_65); -x_70 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_340____closed__1; +x_70 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379____closed__1; x_71 = l_Lean_Linter_UnusedVariables_visitAssignments___closed__1; x_72 = l_Lean_Linter_UnusedVariables_visitAssignments___closed__3; x_73 = lean_box(0); -x_74 = l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___lambda__1(x_63, x_70, x_3, x_1, x_4, x_5, x_71, x_72, x_10, x_73, x_7, x_8, x_64); +x_74 = l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___lambda__1(x_63, x_70, x_3, x_1, x_4, x_5, x_71, x_10, x_72, x_73, x_7, x_8, x_64); return x_74; } else @@ -19131,7 +21048,7 @@ else size_t x_28; size_t x_29; lean_object* x_30; x_28 = 0; x_29 = lean_usize_of_nat(x_18); -x_30 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26(x_17, x_28, x_29, x_3, x_4, x_13); +x_30 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__32(x_17, x_28, x_29, x_3, x_4, x_13); if (lean_obj_tag(x_30) == 0) { lean_object* x_31; lean_object* x_32; uint8_t x_33; @@ -19371,7 +21288,7 @@ static lean_object* _init_l_Lean_Linter_UnusedVariables_unusedVariables___closed lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__8; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__11; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__11; x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__2; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; @@ -19414,20 +21331,31 @@ lean_dec(x_2); return x_5; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__3___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__3(x_1, x_2, x_3); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__4___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__3(x_1, x_2); +x_3 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__4(x_1, x_2); lean_dec(x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; -x_7 = l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); @@ -19436,11 +21364,11 @@ lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; -x_9 = l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); @@ -19463,18 +21391,7 @@ x_10 = lean_box(x_9); return x_10; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__11(x_1, x_2, x_3); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_4; -} -} -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__12___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { size_t x_7; size_t x_8; uint8_t x_9; lean_object* x_10; @@ -19482,7 +21399,7 @@ x_7 = lean_unbox_usize(x_5); lean_dec(x_5); x_8 = lean_unbox_usize(x_6); lean_dec(x_6); -x_9 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__12(x_1, x_2, x_3, x_4, x_7, x_8); +x_9 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__11(x_1, x_2, x_3, x_4, x_7, x_8); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); @@ -19491,17 +21408,47 @@ x_10 = lean_box(x_9); return x_10; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__14___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_5; -x_5 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__13(x_1, x_2, x_3, x_4); +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); lean_dec(x_2); +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__14(x_1, x_5, x_6, x_4); lean_dec(x_1); -return x_5; +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15(x_1, x_2, x_3, x_7, x_8, x_6); +lean_dec(x_3); +lean_dec(x_2); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16(x_1, x_5, x_6, x_4); +lean_dec(x_1); +return x_7; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__14___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__17___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { size_t x_7; size_t x_8; lean_object* x_9; @@ -19509,35 +21456,74 @@ x_7 = lean_unbox_usize(x_4); lean_dec(x_4); x_8 = lean_unbox_usize(x_5); lean_dec(x_5); -x_9 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__14(x_1, x_2, x_3, x_7, x_8, x_6); +x_9 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__17(x_1, x_2, x_3, x_7, x_8, x_6); +lean_dec(x_3); +lean_dec(x_2); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__18___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = lean_unbox_usize(x_3); lean_dec(x_3); +x_7 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__18(x_1, x_5, x_6, x_4); +lean_dec(x_1); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); lean_dec(x_2); +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19(x_1, x_5, x_6, x_4); lean_dec(x_1); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20(x_1, x_2, x_3, x_7, x_8, x_6); +lean_dec(x_3); +lean_dec(x_2); return x_9; } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___lambda__1(x_1, x_2); +x_3 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___lambda__1(x_1, x_2); lean_dec(x_2); lean_dec(x_1); x_4 = lean_box(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { uint8_t x_7; lean_object* x_8; -x_7 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_3); x_8 = lean_box(x_7); return x_8; } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { size_t x_12; size_t x_13; lean_object* x_14; @@ -19545,23 +21531,23 @@ x_12 = lean_unbox_usize(x_7); lean_dec(x_7); x_13 = lean_unbox_usize(x_8); lean_dec(x_8); -x_14 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15(x_1, x_2, x_3, x_4, x_5, x_6, x_12, x_13, x_9, x_10, x_11); +x_14 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21(x_1, x_2, x_3, x_4, x_5, x_6, x_12, x_13, x_9, x_10, x_11); lean_dec(x_6); return x_14; } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16___lambda__1(x_1, x_2); +x_3 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___lambda__1(x_1, x_2); lean_dec(x_2); lean_dec(x_1); x_4 = lean_box(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { size_t x_12; size_t x_13; lean_object* x_14; @@ -19569,12 +21555,12 @@ x_12 = lean_unbox_usize(x_7); lean_dec(x_7); x_13 = lean_unbox_usize(x_8); lean_dec(x_8); -x_14 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16(x_1, x_2, x_3, x_4, x_5, x_6, x_12, x_13, x_9, x_10, x_11); +x_14 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22(x_1, x_2, x_3, x_4, x_5, x_6, x_12, x_13, x_9, x_10, x_11); lean_dec(x_6); return x_14; } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__17___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__23___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { size_t x_7; size_t x_8; uint8_t x_9; lean_object* x_10; @@ -19582,13 +21568,13 @@ x_7 = lean_unbox_usize(x_5); lean_dec(x_5); x_8 = lean_unbox_usize(x_6); lean_dec(x_6); -x_9 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__17(x_1, x_2, x_3, x_4, x_7, x_8); +x_9 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__23(x_1, x_2, x_3, x_4, x_7, x_8); lean_dec(x_4); x_10 = lean_box(x_9); return x_10; } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__18___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__24___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { size_t x_7; size_t x_8; uint8_t x_9; lean_object* x_10; @@ -19596,7 +21582,7 @@ x_7 = lean_unbox_usize(x_5); lean_dec(x_5); x_8 = lean_unbox_usize(x_6); lean_dec(x_6); -x_9 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__18(x_1, x_2, x_3, x_4, x_7, x_8); +x_9 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__24(x_1, x_2, x_3, x_4, x_7, x_8); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); @@ -19605,47 +21591,65 @@ x_10 = lean_box(x_9); return x_10; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__1___boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__1___boxed(lean_object* x_1) { _start: { uint8_t x_2; lean_object* x_3; -x_2 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__1(x_1); +x_2 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__1(x_1); lean_dec(x_1); x_3 = lean_box(x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { uint8_t x_9; lean_object* x_10; x_9 = lean_unbox(x_3); lean_dec(x_3); -x_10 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__2(x_1, x_2, x_9, x_4, x_5, x_6, x_7, x_8); +x_10 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__2(x_1, x_2, x_9, x_4, x_5, x_6, x_7, x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); return x_10; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__3___boxed(lean_object** _args) { +lean_object* x_1 = _args[0]; +lean_object* x_2 = _args[1]; +lean_object* x_3 = _args[2]; +lean_object* x_4 = _args[3]; +lean_object* x_5 = _args[4]; +lean_object* x_6 = _args[5]; +lean_object* x_7 = _args[6]; +lean_object* x_8 = _args[7]; +lean_object* x_9 = _args[8]; +lean_object* x_10 = _args[9]; +lean_object* x_11 = _args[10]; +lean_object* x_12 = _args[11]; +lean_object* x_13 = _args[12]; +lean_object* x_14 = _args[13]; +lean_object* x_15 = _args[14]; +lean_object* x_16 = _args[15]; +lean_object* x_17 = _args[16]; _start: { -uint8_t x_16; lean_object* x_17; -x_16 = lean_unbox(x_10); -lean_dec(x_10); -x_17 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_16, x_11, x_12, x_13, x_14, x_15); -lean_dec(x_14); -lean_dec(x_13); +uint8_t x_18; lean_object* x_19; +x_18 = lean_unbox(x_12); lean_dec(x_12); +x_19 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_18, x_13, x_14, x_15, x_16, x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); -return x_17; +return x_19; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__4___boxed(lean_object** _args) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__4___boxed(lean_object** _args) { lean_object* x_1 = _args[0]; lean_object* x_2 = _args[1]; lean_object* x_3 = _args[2]; @@ -19667,25 +21671,28 @@ lean_object* x_18 = _args[17]; lean_object* x_19 = _args[18]; lean_object* x_20 = _args[19]; lean_object* x_21 = _args[20]; +lean_object* x_22 = _args[21]; +lean_object* x_23 = _args[22]; _start: { -uint8_t x_22; uint8_t x_23; lean_object* x_24; -x_22 = lean_unbox(x_10); -lean_dec(x_10); -x_23 = lean_unbox(x_16); -lean_dec(x_16); -x_24 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_22, x_11, x_12, x_13, x_14, x_15, x_23, x_17, x_18, x_19, x_20, x_21); +uint8_t x_24; uint8_t x_25; lean_object* x_26; +x_24 = lean_unbox(x_12); +lean_dec(x_12); +x_25 = lean_unbox(x_18); lean_dec(x_18); -lean_dec(x_15); -lean_dec(x_11); +x_26 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_24, x_13, x_14, x_15, x_16, x_17, x_25, x_19, x_20, x_21, x_22, x_23); +lean_dec(x_20); +lean_dec(x_17); +lean_dec(x_13); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); -return x_24; +return x_26; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__5___boxed(lean_object** _args) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__5___boxed(lean_object** _args) { lean_object* x_1 = _args[0]; lean_object* x_2 = _args[1]; lean_object* x_3 = _args[2]; @@ -19708,25 +21715,28 @@ lean_object* x_19 = _args[18]; lean_object* x_20 = _args[19]; lean_object* x_21 = _args[20]; lean_object* x_22 = _args[21]; +lean_object* x_23 = _args[22]; +lean_object* x_24 = _args[23]; _start: { -uint8_t x_23; uint8_t x_24; lean_object* x_25; -x_23 = lean_unbox(x_12); -lean_dec(x_12); -x_24 = lean_unbox(x_17); -lean_dec(x_17); -x_25 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_23, x_13, x_14, x_15, x_16, x_24, x_18, x_19, x_20, x_21, x_22); +uint8_t x_25; uint8_t x_26; lean_object* x_27; +x_25 = lean_unbox(x_14); +lean_dec(x_14); +x_26 = lean_unbox(x_19); lean_dec(x_19); -lean_dec(x_16); -lean_dec(x_13); +x_27 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_25, x_15, x_16, x_17, x_18, x_26, x_20, x_21, x_22, x_23, x_24); +lean_dec(x_21); +lean_dec(x_18); +lean_dec(x_15); +lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_6); -return x_25; +return x_27; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__6___boxed(lean_object** _args) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__6___boxed(lean_object** _args) { lean_object* x_1 = _args[0]; lean_object* x_2 = _args[1]; lean_object* x_3 = _args[2]; @@ -19749,24 +21759,27 @@ lean_object* x_19 = _args[18]; lean_object* x_20 = _args[19]; lean_object* x_21 = _args[20]; lean_object* x_22 = _args[21]; +lean_object* x_23 = _args[22]; +lean_object* x_24 = _args[23]; _start: { -uint8_t x_23; uint8_t x_24; lean_object* x_25; -x_23 = lean_unbox(x_12); -lean_dec(x_12); -x_24 = lean_unbox(x_17); -lean_dec(x_17); -x_25 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_23, x_13, x_14, x_15, x_16, x_24, x_18, x_19, x_20, x_21, x_22); +uint8_t x_25; uint8_t x_26; lean_object* x_27; +x_25 = lean_unbox(x_14); +lean_dec(x_14); +x_26 = lean_unbox(x_19); lean_dec(x_19); -lean_dec(x_16); -lean_dec(x_13); +x_27 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_25, x_15, x_16, x_17, x_18, x_26, x_20, x_21, x_22, x_23, x_24); +lean_dec(x_21); +lean_dec(x_18); +lean_dec(x_15); +lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -return x_25; +return x_27; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___boxed(lean_object** _args) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___boxed(lean_object** _args) { lean_object* x_1 = _args[0]; lean_object* x_2 = _args[1]; lean_object* x_3 = _args[2]; @@ -19785,55 +21798,60 @@ lean_object* x_15 = _args[14]; lean_object* x_16 = _args[15]; lean_object* x_17 = _args[16]; lean_object* x_18 = _args[17]; +lean_object* x_19 = _args[18]; +lean_object* x_20 = _args[19]; +lean_object* x_21 = _args[20]; _start: { -uint8_t x_19; size_t x_20; size_t x_21; lean_object* x_22; -x_19 = lean_unbox(x_4); +uint8_t x_22; size_t x_23; size_t x_24; lean_object* x_25; +x_22 = lean_unbox(x_4); lean_dec(x_4); -x_20 = lean_unbox_usize(x_13); -lean_dec(x_13); -x_21 = lean_unbox_usize(x_14); -lean_dec(x_14); -x_22 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19(x_1, x_2, x_3, x_19, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_20, x_21, x_15, x_16, x_17, x_18); +x_23 = lean_unbox_usize(x_16); +lean_dec(x_16); +x_24 = lean_unbox_usize(x_17); +lean_dec(x_17); +x_25 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25(x_1, x_2, x_3, x_22, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_23, x_24, x_18, x_19, x_20, x_21); +lean_dec(x_15); lean_dec(x_12); -lean_dec(x_9); +lean_dec(x_11); +lean_dec(x_10); lean_dec(x_8); lean_dec(x_3); lean_dec(x_2); -return x_22; +return x_25; } } -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1(x_1, x_2); +x_3 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1(x_1, x_2); lean_dec(x_2); lean_dec(x_1); x_4 = lean_box(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20(x_1, x_2, x_3); +x_4 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26(x_1, x_2, x_3); lean_dec(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; -x_7 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_5); lean_dec(x_2); return x_7; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { size_t x_8; size_t x_9; lean_object* x_10; @@ -19841,13 +21859,13 @@ x_8 = lean_unbox_usize(x_2); lean_dec(x_2); x_9 = lean_unbox_usize(x_3); lean_dec(x_3); -x_10 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22(x_1, x_8, x_9, x_4, x_5, x_6, x_7); +x_10 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28(x_1, x_8, x_9, x_4, x_5, x_6, x_7); lean_dec(x_6); lean_dec(x_1); return x_10; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__23___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__29___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { size_t x_5; size_t x_6; lean_object* x_7; @@ -19855,12 +21873,12 @@ x_5 = lean_unbox_usize(x_2); lean_dec(x_2); x_6 = lean_unbox_usize(x_3); lean_dec(x_3); -x_7 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__23(x_1, x_5, x_6, x_4); +x_7 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__29(x_1, x_5, x_6, x_4); lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__24___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__30___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { size_t x_5; size_t x_6; lean_object* x_7; @@ -19868,12 +21886,12 @@ x_5 = lean_unbox_usize(x_2); lean_dec(x_2); x_6 = lean_unbox_usize(x_3); lean_dec(x_3); -x_7 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__24(x_1, x_5, x_6, x_4); +x_7 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__30(x_1, x_5, x_6, x_4); lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__31___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { size_t x_7; size_t x_8; lean_object* x_9; @@ -19881,13 +21899,13 @@ x_7 = lean_unbox_usize(x_4); lean_dec(x_4); x_8 = lean_unbox_usize(x_5); lean_dec(x_5); -x_9 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25(x_1, x_2, x_3, x_7, x_8, x_6); +x_9 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__31(x_1, x_2, x_3, x_7, x_8, x_6); lean_dec(x_3); lean_dec(x_2); return x_9; } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__32___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { size_t x_7; size_t x_8; lean_object* x_9; @@ -19895,7 +21913,7 @@ x_7 = lean_unbox_usize(x_2); lean_dec(x_2); x_8 = lean_unbox_usize(x_3); lean_dec(x_3); -x_9 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26(x_1, x_7, x_8, x_4, x_5, x_6); +x_9 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__32(x_1, x_7, x_8, x_4, x_5, x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_1); @@ -19946,7 +21964,7 @@ lean_dec(x_2); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_initFn____x40_Lean_Linter_UnusedVariables___hyg_5794_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_initFn____x40_Lean_Linter_UnusedVariables___hyg_6304_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; @@ -20069,6 +22087,21 @@ if (lean_io_result_is_error(res)) return res; l_Lean_Linter_linter_unusedVariables_patternVars = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Linter_linter_unusedVariables_patternVars); lean_dec_ref(res); +}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__4(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__4); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__5(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__5); +if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125_(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +l_Lean_Linter_linter_unusedVariables_analyzeTactics = lean_io_result_get_value(res); +lean_mark_persistent(l_Lean_Linter_linter_unusedVariables_analyzeTactics); +lean_dec_ref(res); }l_Lean_Linter_getLinterUnusedVariables___closed__1 = _init_l_Lean_Linter_getLinterUnusedVariables___closed__1(); lean_mark_persistent(l_Lean_Linter_getLinterUnusedVariables___closed__1); l_Lean_Linter_mkIgnoreFnImpl___closed__1 = _init_l_Lean_Linter_mkIgnoreFnImpl___closed__1(); @@ -20085,418 +22118,418 @@ l_Lean_Linter_mkIgnoreFnImpl___closed__6 = _init_l_Lean_Linter_mkIgnoreFnImpl___ lean_mark_persistent(l_Lean_Linter_mkIgnoreFnImpl___closed__6); l_Lean_Linter_mkIgnoreFnImpl___closed__7 = _init_l_Lean_Linter_mkIgnoreFnImpl___closed__7(); lean_mark_persistent(l_Lean_Linter_mkIgnoreFnImpl___closed__7); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_340____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_340____closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_340____closed__1); -if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_340_(lean_io_mk_world()); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379____closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379____closed__1); +if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_Linter_builtinUnusedVariablesIgnoreFnsRef = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Linter_builtinUnusedVariablesIgnoreFnsRef); lean_dec_ref(res); }l_Lean_Linter_addBuiltinUnusedVariablesIgnoreFn___closed__1 = _init_l_Lean_Linter_addBuiltinUnusedVariablesIgnoreFn___closed__1(); lean_mark_persistent(l_Lean_Linter_addBuiltinUnusedVariablesIgnoreFn___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__3(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__3); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__4(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__4); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__5(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__5); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__6(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__6); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__7(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__7); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__8(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__8); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__9(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__9); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__10 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__10(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__10); -if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387_(lean_io_mk_world()); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__4(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__4); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__5(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__5); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__6(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__6); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__7(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__7); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__8(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__8); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__9(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__9); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__10 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__10(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__10); +if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_Linter_unusedVariablesIgnoreFnsExt = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Linter_unusedVariablesIgnoreFnsExt); lean_dec_ref(res); -}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__3); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__3(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__3); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__5___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__5___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__5___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__3(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__3); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__4(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__4); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__5(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__5); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__6(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__6); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__7(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__7); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__8(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__8); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__9(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__9); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__10 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__10(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__10); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__11 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__11(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__11); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__12 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__12(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__12); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__13 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__13(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__13); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__14 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__14(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__14); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__15 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__15(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__15); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__16 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__16(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__16); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__17 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__17(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__17); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__18 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__18(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__18); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__19 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__19(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__19); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__20 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__20(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__20); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__21 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__21(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__21); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__22 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__22(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__22); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__23 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__23(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__23); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__24 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__24(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__24); -if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601_(lean_io_mk_world()); +}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__5___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__5___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__5___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__4(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__4); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__5(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__5); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__6(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__6); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__7(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__7); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__8(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__8); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__9(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__9); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__10 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__10(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__10); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__11 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__11(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__11); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__12 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__12(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__12); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__13 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__13(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__13); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__14 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__14(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__14); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__15 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__15(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__15); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__16 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__16(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__16); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__17 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__17(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__17); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__18 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__18(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__18); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__19 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__19(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__19); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__20 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__20(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__20); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__21 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__21(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__21); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__22 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__22(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__22); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__23 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__23(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__23); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__24 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__24(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__24); +if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__6(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__6); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__7(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__7); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__8(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__8); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__9(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__9); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__10 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__10(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__10); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__11 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__11(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__11); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__12 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__12(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__12); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____closed__1); -if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948_(lean_io_mk_world()); +}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__6); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__7(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__7); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__8(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__8); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__9(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__9); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__10 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__10(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__10); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__11 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__11(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__11); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__12 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__12(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__12); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____closed__1); +if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__3); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__4); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__5(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__5); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__6(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__6); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__7(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__7); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____closed__1); -if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982_(lean_io_mk_world()); +}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__4); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__5); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__6); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__7(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__7); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____closed__1); +if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__3); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__4); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__5(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__5); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__6(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__6); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__7(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__7); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__8(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__8); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__9(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__9); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__10 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__10(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__10); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__11 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__11(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__11); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__12 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__12(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__12); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__13 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__13(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__13); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__14 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__14(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__14); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____closed__1); -if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016_(lean_io_mk_world()); +}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__4); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__5); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__6); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__7(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__7); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__8(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__8); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__9(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__9); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__10 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__10(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__10); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__11 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__11(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__11); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__12 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__12(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__12); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__13 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__13(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__13); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__14 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__14(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__14); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____closed__1); +if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__3); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__4); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__5(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__5); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__6(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__6); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__7(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__7); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__8(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__8); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__9(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__9); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__10 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__10(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__10); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__11 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__11(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__11); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__12 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__12(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__12); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____closed__1); -if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107_(lean_io_mk_world()); +}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__4); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__5); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__6); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__7(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__7); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__8(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__8); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__9(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__9); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__10 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__10(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__10); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__11 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__11(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__11); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__12 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__12(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__12); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____closed__1); +if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__3); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__4); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__5(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__5); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__6(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__6); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__7(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__7); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__8(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__8); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__9(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__9); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__10 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__10(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__10); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__11 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__11(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__11); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____closed__1); -if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192_(lean_io_mk_world()); +}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__4); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__5); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__6); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__7(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__7); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__8(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__8); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__9(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__9); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__10 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__10(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__10); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__11 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__11(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__11); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____closed__1); +if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__1 = _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__1(); -lean_mark_persistent(l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__1); -l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__2 = _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__2(); -lean_mark_persistent(l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__2); -l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__3 = _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__3(); -lean_mark_persistent(l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__3); -l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__4 = _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__4(); -lean_mark_persistent(l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__4); -l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__5 = _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__5(); -lean_mark_persistent(l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__5); -l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__6 = _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__6(); -lean_mark_persistent(l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__6); -l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__7 = _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__7(); -lean_mark_persistent(l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__7); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__3); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__4); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__5(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__5); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__3(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__3); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__4(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__4); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__5(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__5); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__3(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__3); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__4(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__4); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__5(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__5); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__6(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__6); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__7(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__7); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__8(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__8); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__9(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__9); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__10 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__10(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__10); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__11 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__11(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__11); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__12 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__12(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__12); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__13 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__13(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__13); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____closed__1); -if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277_(lean_io_mk_world()); +}l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__1 = _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__1(); +lean_mark_persistent(l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__1); +l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__2 = _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__2(); +lean_mark_persistent(l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__2); +l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__3 = _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__3(); +lean_mark_persistent(l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__3); +l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__4 = _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__4(); +lean_mark_persistent(l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__4); +l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__5 = _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__5(); +lean_mark_persistent(l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__5); +l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__6 = _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__6(); +lean_mark_persistent(l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__6); +l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__7 = _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__7(); +lean_mark_persistent(l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__7); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__4); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__5); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__4(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__4); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__5(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__5); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__4(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__4); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__5(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__5); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__6(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__6); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__7(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__7); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__8(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__8); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__9(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__9); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__10 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__10(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__10); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__11 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__11(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__11); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__12 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__12(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__12); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__13 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__13(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__13); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____closed__1); +if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__3); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__4); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__5(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__5); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__6(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__6); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__7(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__7); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__8(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__8); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__9(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__9); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____closed__1); -if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404_(lean_io_mk_world()); +}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__4); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__5); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__6); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__7(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__7); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__8(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__8); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__9(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__9); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____closed__1); +if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__3); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__4); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__5(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__5); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__6(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__6); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__7(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__7); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__8(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__8); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__9(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__9); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____closed__1); -if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436_(lean_io_mk_world()); +}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__4); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__5); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__6); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__7(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__7); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__8(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__8); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__9(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__9); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____closed__1); +if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__3); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____closed__1); -if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555_(lean_io_mk_world()); +}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____closed__1); +if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__3); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__4); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__5(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__5); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__6(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__6); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__7(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__7); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__8(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__8); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__9(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__9); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____closed__1); -if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651_(lean_io_mk_world()); +}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__4); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__5); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__6); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__7(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__7); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__8(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__8); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__9(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__9); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____closed__1); +if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__3); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__4); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__5(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__5); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__2___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__2___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__2___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____closed__1); -if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703_(lean_io_mk_world()); +}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__4); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__5); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__2___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__2___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____closed__1); +if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l_Lean_Linter_getUnusedVariablesIgnoreFns___rarg___closed__1 = _init_l_Lean_Linter_getUnusedVariablesIgnoreFns___rarg___closed__1(); @@ -20511,70 +22544,89 @@ l_Lean_Linter_UnusedVariables_collectReferences_skipDeclIdIfPresent___closed__1 lean_mark_persistent(l_Lean_Linter_UnusedVariables_collectReferences_skipDeclIdIfPresent___closed__1); l_Lean_Linter_UnusedVariables_collectReferences_skipDeclIdIfPresent___closed__2 = _init_l_Lean_Linter_UnusedVariables_collectReferences_skipDeclIdIfPresent___closed__2(); lean_mark_persistent(l_Lean_Linter_UnusedVariables_collectReferences_skipDeclIdIfPresent___closed__2); -l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__1 = _init_l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__1(); -lean_mark_persistent(l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__1); -l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__2 = _init_l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__2(); -lean_mark_persistent(l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__2); -l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__3 = _init_l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__3(); -lean_mark_persistent(l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__3); -l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__1 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__1(); -lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__1); -l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__2 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__2(); -lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__2); -l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__3 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__3(); -lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__3); -l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__4 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__4(); -lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__4); -l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__1); -l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__2 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__2(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__2); -l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__3 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__3(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__3); -l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__4 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__4(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__4); -l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___closed__1); +l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14___closed__1 = _init_l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14___closed__1(); +lean_mark_persistent(l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14___closed__1); +l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__1 = _init_l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__1(); +lean_mark_persistent(l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__1); +l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__2 = _init_l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__2(); +lean_mark_persistent(l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__2); +l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__3 = _init_l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__3(); +lean_mark_persistent(l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__3); +l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__4 = _init_l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__4(); +lean_mark_persistent(l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__4); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__1 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__1(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__1); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__2 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__2(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__2); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__3 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__3(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__3); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__4 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__4(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__4); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__1(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__1); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__2 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__2(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__2); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__3 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__3(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__3); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__4 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__4(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__4); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__7___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__7___closed__1(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__7___closed__1); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__1(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__1); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__2 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__2(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__2); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__3 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__3(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__3); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__4 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__4(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__4); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__5 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__5(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__5); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__6 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__6(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__6); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___closed__1(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___closed__1); l_panic___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__8___closed__1 = _init_l_panic___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__8___closed__1(); lean_mark_persistent(l_panic___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__8___closed__1); -l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___lambda__2___closed__1 = _init_l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___lambda__2___closed__1(); -lean_mark_persistent(l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___lambda__2___closed__1); -l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___closed__1 = _init_l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___closed__1(); -lean_mark_persistent(l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___closed__1); -l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__5___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__5___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__5___closed__1); -l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__1 = _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__1(); -lean_mark_persistent(l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__1); -l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__2 = _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__2(); -lean_mark_persistent(l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__2); -l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__3 = _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__3(); -lean_mark_persistent(l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__3); -l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__4 = _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__4(); -lean_mark_persistent(l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__4); -l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___closed__1 = _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___closed__1(); -lean_mark_persistent(l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___closed__1); -l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__1 = _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__1(); -lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__1); -l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__2 = _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__2(); -lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__2); -l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__3 = _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__3(); -lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__3); -l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__4 = _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__4(); -lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__4); -l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__5 = _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__5(); -lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__5); -l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__6 = _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__6(); -lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__6); -l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__7 = _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__7(); -lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__7); -l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__1); -l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__2 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__2(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__2); -l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__3 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__3(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__3); -l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__4 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__4(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__4); +l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___lambda__2___closed__1 = _init_l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___lambda__2___closed__1); +l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___closed__1 = _init_l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___closed__1(); +lean_mark_persistent(l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___closed__1); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__3___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__3___closed__1(); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__5___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__5___closed__1(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__5___closed__1); +l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__1 = _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__1(); +lean_mark_persistent(l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__1); +l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__2 = _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__2(); +lean_mark_persistent(l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__2); +l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__3 = _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__3(); +lean_mark_persistent(l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__3); +l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__4 = _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__4(); +lean_mark_persistent(l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__4); +l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___closed__1 = _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___closed__1(); +lean_mark_persistent(l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___closed__1); +l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__1 = _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__1(); +lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__1); +l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__2 = _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__2(); +lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__2); +l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__3 = _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__3(); +lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__3); +l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__4 = _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__4(); +lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__4); +l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__5 = _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__5(); +lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__5); +l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__6 = _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__6(); +lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__6); +l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__7 = _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__7(); +lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__7); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__1(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__1); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__2 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__2(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__2); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__3 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__3(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__3); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__4 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__4(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__4); l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___lambda__2___closed__1 = _init_l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___lambda__2___closed__1(); lean_mark_persistent(l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___lambda__2___closed__1); l_Lean_Linter_UnusedVariables_unusedVariables___closed__1 = _init_l_Lean_Linter_UnusedVariables_unusedVariables___closed__1(); @@ -20585,7 +22637,7 @@ l_Lean_Linter_UnusedVariables_unusedVariables___closed__3 = _init_l_Lean_Linter_ lean_mark_persistent(l_Lean_Linter_UnusedVariables_unusedVariables___closed__3); l_Lean_Linter_UnusedVariables_unusedVariables = _init_l_Lean_Linter_UnusedVariables_unusedVariables(); lean_mark_persistent(l_Lean_Linter_UnusedVariables_unusedVariables); -if (builtin) {res = l_Lean_Linter_UnusedVariables_initFn____x40_Lean_Linter_UnusedVariables___hyg_5794_(lean_io_mk_world()); +if (builtin) {res = l_Lean_Linter_UnusedVariables_initFn____x40_Lean_Linter_UnusedVariables___hyg_6304_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l_Lean_MessageData_isUnusedVariableWarning___closed__1 = _init_l_Lean_MessageData_isUnusedVariableWarning___closed__1(); diff --git a/stage0/stdlib/Lean/Linter/Util.c b/stage0/stdlib/Lean/Linter/Util.c index af3e5c0d410e..38871709e0b5 100644 --- a/stage0/stdlib/Lean/Linter/Util.c +++ b/stage0/stdlib/Lean/Linter/Util.c @@ -13,26 +13,44 @@ #ifdef __cplusplus extern "C" { #endif +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3(lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go(lean_object*); -lean_object* l_Lean_Elab_InfoTree_visitM_go___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__5___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_PersistentArray_toList___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___lambda__1(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__4; LEAN_EXPORT lean_object* l_List_filterMapTR_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__2___closed__2; +lean_object* l_Lean_Elab_Info_updateContext_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f___rarg___lambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__5(lean_object*); +lean_object* l_Lean_Elab_PartialContextInfo_mergeIntoOuter_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterMapTR_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__2(lean_object*, lean_object*); lean_object* lean_array_to_list(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3(lean_object*); +lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__3; LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__2; +LEAN_EXPORT lean_object* l_panic___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__4(lean_object*); +lean_object* lean_panic_fn(lean_object*, lean_object*); lean_object* l_List_reverse___rarg(lean_object*); +LEAN_EXPORT lean_object* l_panic___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__4___rarg(lean_object*, lean_object*); lean_object* lean_array_mk(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_instInhabitedOfMonad___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__5___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Elab_Info_contains(lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_List_filterMapTR_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__1(lean_object* x_1, lean_object* x_2) { _start: @@ -114,36 +132,328 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_panic___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__4___rarg(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_5; lean_object* x_6; -x_5 = lean_box(0); -x_6 = l_Lean_Elab_InfoTree_visitM_go___rarg(x_1, x_2, x_3, x_5, x_4); +lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_3 = lean_box(0); +x_4 = l_instInhabitedOfMonad___rarg(x_1, x_3); +x_5 = lean_panic_fn(x_4, x_2); +return x_5; +} +} +LEAN_EXPORT lean_object* l_panic___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__4(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_panic___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__4___rarg), 2, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__5___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; lean_object* x_9; +x_8 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_8, 0, x_7); +lean_ctor_set(x_8, 1, x_1); +x_9 = l_List_mapM_loop___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__5___rarg(x_2, x_3, x_4, x_5, x_6, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__5___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = l_List_reverse___rarg(x_6); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_11 = lean_ctor_get(x_5, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_5, 1); +lean_inc(x_12); +lean_dec(x_5); +x_13 = lean_ctor_get(x_1, 1); +lean_inc(x_13); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg(x_1, x_2, x_3, x_4, x_11); +x_15 = lean_alloc_closure((void*)(l_List_mapM_loop___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__5___rarg___lambda__1), 7, 6); +lean_closure_set(x_15, 0, x_6); +lean_closure_set(x_15, 1, x_1); +lean_closure_set(x_15, 2, x_2); +lean_closure_set(x_15, 3, x_3); +lean_closure_set(x_15, 4, x_4); +lean_closure_set(x_15, 5, x_12); +x_16 = lean_apply_4(x_13, lean_box(0), lean_box(0), x_14, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__5(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_List_mapM_loop___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__5___rarg), 6, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___lambda__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_3 = lean_ctor_get(x_1, 0); +lean_inc(x_3); +lean_dec(x_1); +x_4 = lean_ctor_get(x_3, 1); +lean_inc(x_4); +lean_dec(x_3); +x_5 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_5, 0, x_2); +x_6 = lean_apply_2(x_4, lean_box(0), x_5); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_8 = lean_apply_4(x_1, x_2, x_3, x_4, x_7); +x_9 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___lambda__1), 2, 1); +lean_closure_set(x_9, 0, x_5); +x_10 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, uint8_t x_8) { +_start: +{ +if (x_8 == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +lean_dec(x_7); +x_9 = lean_box(0); +x_10 = lean_apply_4(x_1, x_2, x_3, x_4, x_9); +x_11 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___lambda__1), 2, 1); +lean_closure_set(x_11, 0, x_5); +x_12 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_10, x_11); +return x_12; +} +else +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +lean_inc(x_2); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_2); +x_14 = l_Lean_Elab_Info_updateContext_x3f(x_13, x_3); +x_15 = l_Lean_PersistentArray_toList___rarg(x_4); +x_16 = lean_box(0); +lean_inc(x_1); +lean_inc(x_5); +x_17 = l_List_mapM_loop___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__5___rarg(x_5, x_7, x_1, x_14, x_15, x_16); +lean_inc(x_6); +x_18 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___lambda__2), 7, 6); +lean_closure_set(x_18, 0, x_1); +lean_closure_set(x_18, 1, x_2); +lean_closure_set(x_18, 2, x_3); +lean_closure_set(x_18, 3, x_4); +lean_closure_set(x_18, 4, x_5); +lean_closure_set(x_18, 5, x_6); +x_19 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_17, x_18); +return x_19; +} +} +} +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean.Server.InfoUtils", 21, 21); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean.Elab.InfoTree.visitM.go", 28, 28); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("unexpected context-free info tree node", 38, 38); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__1; +x_2 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__2; +x_3 = lean_unsigned_to_nat(62u); +x_4 = lean_unsigned_to_nat(21u); +x_5 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__3; +x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_4) == 0) +{ +switch (lean_obj_tag(x_5)) { +case 0: +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_6 = lean_ctor_get(x_5, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_5, 1); +lean_inc(x_7); +lean_dec(x_5); +x_8 = l_Lean_Elab_PartialContextInfo_mergeIntoOuter_x3f(x_6, x_4); +x_4 = x_8; +x_5 = x_7; +goto _start; +} +case 1: +{ +lean_object* x_10; lean_object* x_11; +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +x_10 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__4; +x_11 = l_panic___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__4___rarg(x_1, x_10); +return x_11; +} +default: +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +x_12 = lean_ctor_get(x_1, 0); +lean_inc(x_12); +lean_dec(x_1); +x_13 = lean_ctor_get(x_12, 1); +lean_inc(x_13); +lean_dec(x_12); +x_14 = lean_box(0); +x_15 = lean_apply_2(x_13, lean_box(0), x_14); +return x_15; +} +} +} +else +{ +switch (lean_obj_tag(x_5)) { +case 0: +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_5, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_5, 1); +lean_inc(x_17); +lean_dec(x_5); +x_18 = l_Lean_Elab_PartialContextInfo_mergeIntoOuter_x3f(x_16, x_4); +x_4 = x_18; +x_5 = x_17; +goto _start; +} +case 1: +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_20 = lean_ctor_get(x_4, 0); +lean_inc(x_20); +lean_dec(x_4); +x_21 = lean_ctor_get(x_5, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_5, 1); +lean_inc(x_22); +lean_dec(x_5); +x_23 = lean_ctor_get(x_1, 1); +lean_inc(x_23); +lean_inc(x_2); +lean_inc(x_22); +lean_inc(x_21); +lean_inc(x_20); +x_24 = lean_apply_3(x_2, x_20, x_21, x_22); +lean_inc(x_23); +x_25 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___lambda__3___boxed), 8, 7); +lean_closure_set(x_25, 0, x_3); +lean_closure_set(x_25, 1, x_20); +lean_closure_set(x_25, 2, x_21); +lean_closure_set(x_25, 3, x_22); +lean_closure_set(x_25, 4, x_1); +lean_closure_set(x_25, 5, x_23); +lean_closure_set(x_25, 6, x_2); +x_26 = lean_apply_4(x_23, lean_box(0), lean_box(0), x_24, x_25); +return x_26; +} +default: +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_27 = lean_ctor_get(x_1, 0); +lean_inc(x_27); +lean_dec(x_1); +x_28 = lean_ctor_get(x_27, 1); +lean_inc(x_28); +lean_dec(x_27); +x_29 = lean_box(0); +x_30 = lean_apply_2(x_28, lean_box(0), x_29); +return x_30; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg), 4, 0); +x_2 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg), 5, 0); return x_2; } } LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +lean_object* x_5; lean_object* x_6; uint8_t x_7; lean_object* x_8; lean_object* x_9; x_5 = lean_ctor_get(x_1, 0); lean_inc(x_5); lean_dec(x_1); x_6 = lean_ctor_get(x_5, 1); lean_inc(x_6); lean_dec(x_5); -x_7 = lean_box(0); -x_8 = lean_apply_2(x_6, lean_box(0), x_7); -return x_8; +x_7 = 1; +x_8 = lean_box(x_7); +x_9 = lean_apply_2(x_6, lean_box(0), x_8); +return x_9; } } static lean_object* _init_l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__2___closed__1() { @@ -451,7 +761,7 @@ return x_83; LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_4; lean_object* x_5; lean_object* x_6; +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_inc(x_1); x_4 = lean_alloc_closure((void*)(l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__1___boxed), 4, 1); lean_closure_set(x_4, 0, x_1); @@ -459,8 +769,9 @@ lean_inc(x_1); x_5 = lean_alloc_closure((void*)(l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__2___boxed), 6, 2); lean_closure_set(x_5, 0, x_2); lean_closure_set(x_5, 1, x_1); -x_6 = l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg(x_1, x_4, x_5, x_3); -return x_6; +x_6 = lean_box(0); +x_7 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg(x_1, x_4, x_5, x_6, x_3); +return x_7; } } LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go(lean_object* x_1) { @@ -471,6 +782,16 @@ x_2 = lean_alloc_closure((void*)(l_Lean_Linter_collectMacroExpansions_x3f_go___r return x_2; } } +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +uint8_t x_9; lean_object* x_10; +x_9 = lean_unbox(x_8); +lean_dec(x_8); +x_10 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_9); +return x_10; +} +} LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { @@ -608,6 +929,14 @@ lean_dec_ref(res); res = initialize_Lean_Linter_Basic(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__1 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__1(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__1); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__2 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__2(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__2); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__3 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__3(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__3); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__4 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__4(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__4); l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__2___closed__1 = _init_l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__2___closed__1(); lean_mark_persistent(l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__2___closed__1); l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__2___closed__2 = _init_l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__2___closed__2(); diff --git a/stage0/stdlib/Lean/Message.c b/stage0/stdlib/Lean/Message.c index 5335c1dfbb1a..19f649ef27b6 100644 --- a/stage0/stdlib/Lean/Message.c +++ b/stage0/stdlib/Lean/Message.c @@ -130,6 +130,7 @@ size_t lean_usize_of_nat(lean_object*); static lean_object* l_Lean_instBEqMessageSeverity___closed__1; LEAN_EXPORT lean_object* l_Lean_stringToMessageData(lean_object*); lean_object* l_Lean_Expr_mvar___override(lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_MessageData_instCoeListExpr(lean_object*); lean_object* l_Lean_instInhabitedPersistentArrayNode(lean_object*); static lean_object* l_Lean_MessageData_formatAux___lambda__1___closed__6; @@ -326,7 +327,6 @@ LEAN_EXPORT lean_object* l_Lean_MessageData_nestD(lean_object*); static lean_object* l___private_Lean_Message_0__Lean_fromJsonMessageSeverity____x40_Lean_Message___hyg_163____lambda__2___closed__1; LEAN_EXPORT lean_object* l_panic___at_Lean_MessageData_formatAux___spec__2(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_MessageLog_hasErrors___spec__3(lean_object*, size_t, size_t); -lean_object* l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Message_0__Lean_fromJsonMessageSeverity____x40_Lean_Message___hyg_163____lambda__3___closed__1; LEAN_EXPORT uint8_t l_Lean_PersistentArray_anyM___at_Lean_MessageLog_hasErrors___spec__1(lean_object*); double l_Float_ofScientific(lean_object*, uint8_t, lean_object*); @@ -5474,7 +5474,7 @@ x_42 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_42, 0, x_14); lean_ctor_set(x_42, 1, x_41); x_43 = l___private_Lean_Message_0__Lean_fromJsonMessageSeverity____x40_Lean_Message___hyg_163____closed__1; -x_44 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_42, x_43); +x_44 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_42, x_43); x_45 = l_Lean_Json_mkObj(x_44); return x_45; } @@ -5502,7 +5502,7 @@ x_53 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_53, 0, x_14); lean_ctor_set(x_53, 1, x_52); x_54 = l___private_Lean_Message_0__Lean_fromJsonMessageSeverity____x40_Lean_Message___hyg_163____closed__1; -x_55 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_53, x_54); +x_55 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_53, x_54); x_56 = l_Lean_Json_mkObj(x_55); return x_56; } @@ -7212,7 +7212,7 @@ x_45 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_45, 0, x_17); lean_ctor_set(x_45, 1, x_44); x_46 = l___private_Lean_Message_0__Lean_fromJsonMessageSeverity____x40_Lean_Message___hyg_163____closed__1; -x_47 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_45, x_46); +x_47 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_45, x_46); x_48 = l_Lean_Json_mkObj(x_47); lean_ctor_set(x_10, 0, x_48); return x_10; @@ -7241,7 +7241,7 @@ x_56 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_56, 0, x_17); lean_ctor_set(x_56, 1, x_55); x_57 = l___private_Lean_Message_0__Lean_fromJsonMessageSeverity____x40_Lean_Message___hyg_163____closed__1; -x_58 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_56, x_57); +x_58 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_56, x_57); x_59 = l_Lean_Json_mkObj(x_58); lean_ctor_set(x_10, 0, x_59); return x_10; @@ -7334,7 +7334,7 @@ x_94 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_94, 0, x_66); lean_ctor_set(x_94, 1, x_93); x_95 = l___private_Lean_Message_0__Lean_fromJsonMessageSeverity____x40_Lean_Message___hyg_163____closed__1; -x_96 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_94, x_95); +x_96 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_94, x_95); x_97 = l_Lean_Json_mkObj(x_96); x_98 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_98, 0, x_97); @@ -7365,7 +7365,7 @@ x_106 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_106, 0, x_66); lean_ctor_set(x_106, 1, x_105); x_107 = l___private_Lean_Message_0__Lean_fromJsonMessageSeverity____x40_Lean_Message___hyg_163____closed__1; -x_108 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_106, x_107); +x_108 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_106, x_107); x_109 = l_Lean_Json_mkObj(x_108); x_110 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_110, 0, x_109); diff --git a/stage0/stdlib/Lean/Meta/AppBuilder.c b/stage0/stdlib/Lean/Meta/AppBuilder.c index c5ed3bc428d9..09f3a1b98986 100644 --- a/stage0/stdlib/Lean/Meta/AppBuilder.c +++ b/stage0/stdlib/Lean/Meta/AppBuilder.c @@ -4191,7 +4191,7 @@ static lean_object* _init_l_Lean_Meta_congrArg_x3f___lambda__4___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_Meta_congrArg_x3f___lambda__4___closed__5; x_2 = l_Lean_Meta_congrArg_x3f___lambda__4___closed__6; -x_3 = lean_unsigned_to_nat(197u); +x_3 = lean_unsigned_to_nat(198u); x_4 = lean_unsigned_to_nat(48u); x_5 = l_Lean_Meta_congrArg_x3f___lambda__4___closed__7; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -4449,7 +4449,7 @@ static lean_object* _init_l_Lean_Meta_congrArg_x3f___closed__3() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_congrArg_x3f___lambda__4___closed__5; x_2 = l_Lean_Meta_congrArg_x3f___lambda__4___closed__6; -x_3 = lean_unsigned_to_nat(194u); +x_3 = lean_unsigned_to_nat(195u); x_4 = lean_unsigned_to_nat(49u); x_5 = l_Lean_Meta_congrArg_x3f___lambda__4___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/Meta/FunInfo.c b/stage0/stdlib/Lean/Meta/FunInfo.c index 6f792e31e3b4..dc78ec55e1a5 100644 --- a/stage0/stdlib/Lean/Meta/FunInfo.c +++ b/stage0/stdlib/Lean/Meta/FunInfo.c @@ -40,16 +40,17 @@ LEAN_EXPORT lean_object* l_Lean_Meta_FunInfo_getArity(lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_fvarId_x21(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Std_Range_forIn_x27_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___lambda__2(lean_object*, lean_object*); lean_object* l_Lean_Meta_forallTelescopeReducing___at_Lean_Meta_getParamNames___spec__2___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isAppOf(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_qsort_sort___at___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_FunInfo_0__Lean_Meta_whenHasVar___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); static size_t l_Lean_PersistentHashMap_findAux___at___private_Lean_Meta_FunInfo_0__Lean_Meta_checkFunInfoCache___spec__2___closed__1; uint64_t l_Lean_Meta_TransparencyMode_hash(uint8_t); @@ -58,7 +59,6 @@ lean_object* lean_st_ref_take(lean_object*, lean_object*); lean_object* l_Lean_getOutParamPositions_x3f(lean_object*, lean_object*); uint8_t lean_expr_eqv(lean_object*, lean_object*); lean_object* l_Lean_Meta_forallBoundedTelescope___at_Lean_Meta_arrowDomainsN___spec__6___rarg(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_getFunInfo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___boxed(lean_object**); LEAN_EXPORT lean_object* l___private_Lean_Meta_FunInfo_0__Lean_Meta_checkFunInfoCache(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1861,7 +1861,7 @@ lean_dec(x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; uint8_t x_9; @@ -1973,7 +1973,7 @@ if (x_5 == 0) lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = lean_array_get_size(x_1); x_7 = lean_mk_empty_array_with_capacity(x_6); -x_8 = l_Array_mapIdxM_map___at___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps___spec__1(x_1, x_2, x_1, x_6, x_4, lean_box(0), x_7); +x_8 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps___spec__1(x_1, x_2, x_1, x_6, x_4, lean_box(0), x_7); return x_8; } else @@ -1983,11 +1983,11 @@ return x_1; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; -x_8 = l_Array_mapIdxM_map___at___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); diff --git a/stage0/stdlib/Lean/Meta/IndPredBelow.c b/stage0/stdlib/Lean/Meta/IndPredBelow.c index ec602eee359b..cb50e528ffff 100644 --- a/stage0/stdlib/Lean/Meta/IndPredBelow.c +++ b/stage0/stdlib/Lean/Meta/IndPredBelow.c @@ -20,8 +20,12 @@ static lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_induction___closed__1; lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_mkCtorType_mkMotiveBinder___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_mkCtorType_mkBelowBinder___spec__3___closed__3; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__7; LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitForall___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__5(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__2; +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__7; lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_visit___spec__3(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_induction(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_IndPredBelow_backwardsChaining___spec__5___lambda__2___closed__8; @@ -30,7 +34,6 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkCt static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__16___rarg___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__9(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_IndPredBelow_mkCtorType_mkBelowBinder___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_checkCount___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_newMotive___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_getConstInfo___at_Lean_Meta_mkConstWithFreshMVarLevels___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -41,7 +44,6 @@ LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_mkCt static lean_object* l_Lean_Meta_IndPredBelow_backwardsChaining___lambda__3___closed__3; static lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow___lambda__3___closed__2; lean_object* l_Lean_commitWhen___at___private_Lean_Meta_Tactic_Contradiction_0__Lean_Meta_elimEmptyInductive___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitPost___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Meta_IndPredBelow_backwardsChaining___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); @@ -50,18 +52,18 @@ lean_object* l_Lean_Meta_mkForallFVars___boxed(lean_object*, lean_object*, lean_ LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkContext_addMotives(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withIncRecDepth___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__15(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_proveBrecOn_applyCtors___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__3; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_rebuild___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_getBelowIndices___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitLambda___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__4___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__2; -static lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__5; static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_6____closed__9; +static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__9; static lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__3___lambda__5___closed__10; static lean_object* l_Std_Range_forIn_loop___at_Lean_Meta_IndPredBelow_mkBelow___spec__1___closed__1; lean_object* lean_whnf(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__16___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__5; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_IndPredBelow_backwardsChaining___spec__5___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitLambda___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__4(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn___closed__3; @@ -69,9 +71,9 @@ static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelo extern lean_object* l_Lean_maxRecDepthErrorMessage; static lean_object* l_Lean_Meta_IndPredBelow_mkBelow___closed__6; uint8_t l_Lean_Exception_isInterrupt(lean_object*); -static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__8; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__2___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__3___lambda__5___closed__6; +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkContext___spec__7(size_t, size_t, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_checkCount___closed__2; lean_object* l_Lean_Meta_isExprDefEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -92,6 +94,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_rebuild(lean_object LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_backwardsChaining(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_findIdx_x3f_loop___rarg(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_sort___override(lean_object*); +static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__8; lean_object* l_Lean_MessageData_ofList(lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__4(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__7___boxed(lean_object*, lean_object*); @@ -106,7 +109,6 @@ static lean_object* l_Lean_getConstInfoInduct___at_Lean_Meta_IndPredBelow_mkCont lean_object* lean_mk_array(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_ST_Prim_Ref_get___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Match_mkMatcher(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_checkCount___lambda__2___closed__1; @@ -121,8 +123,12 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkCt LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_transformFields_loop(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_IndPredBelow_backwardsChaining___spec__5___lambda__2___closed__7; lean_object* l_Lean_Expr_proj___override(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_bvar___override(lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowDecl___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowDecl___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_IndPredBelow_0__Lean_Meta_IndPredBelow_belowType___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__13(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_IndPredBelow_backwardsChaining___spec__5___lambda__2___closed__6; @@ -132,36 +138,32 @@ static lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_checkCount___lambda__1__ lean_object* l_Lean_Meta_ppGoal(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_IndPredBelow_mkContext___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_fvarId_x21(lean_object*); -static lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__1; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkContext___spec__7___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBrecOnDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_getBelowIndices_loop___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowDecl___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__3___lambda__5___closed__4; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_forallTelescopeReducing___at_Lean_Meta_getParamNames___spec__2___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_applyIH___closed__3; static lean_object* l_Lean_Meta_IndPredBelow_mkBelow___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitForall___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__5___lambda__1(lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_addBelowPattern___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_getConstInfoInduct___at_Lean_Meta_IndPredBelow_mkContext___spec__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__7___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_checkCount___closed__3; LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Meta_IndPredBelow_0__Lean_Meta_IndPredBelow_belowType___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__6; -static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__7; lean_object* l_Nat_nextPowerOfTwo_go(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelow(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_stringToMessageData(lean_object*); -static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__9; LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__3___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_backwardsChaining___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_mkContext_motiveType___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__12(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_withLocalDecls___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__8(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__3___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_modifyBinders___lambda__2___boxed(lean_object**); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_closeGoal___closed__7; lean_object* l_Lean_Exception_toMessageData(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_instInhabitedVariables; @@ -176,12 +178,13 @@ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_IndPredBelow_p static lean_object* l_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkIH___closed__2; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_IndPredBelow_backwardsChaining___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Meta_GeneralizeTelescope_generalizeTelescopeAux___spec__1___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkType___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Match_Pattern_toExpr_visit(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_getConstInfoCtor___at___private_Lean_Meta_WHNF_0__Lean_Meta_toCtorWhenStructure___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_instInhabitedNat; static lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__3___lambda__5___closed__8; lean_object* l_List_mapTR_loop___at_Lean_mkConstWithLevelParams___spec__1(lean_object*, lean_object*); -static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__5; +static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__6; LEAN_EXPORT lean_object* l_Lean_getConstInfoInduct___at_Lean_Meta_IndPredBelow_mkContext___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_applyIH(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkConstructor(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -190,7 +193,6 @@ LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_mkBe LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_IndPredBelow_backwardsChaining___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_ptr_addr(lean_object*); lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_appendTR___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__3___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -204,15 +206,15 @@ LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_IndPredBelow_back static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_6____closed__1; static lean_object* l_Lean_Meta_IndPredBelow_backwardsChaining___lambda__3___closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkContext_mkHeader___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkType___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_throwError___at_Lean_Expr_abstractRangeM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__4; +static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__4; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_take(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_IndPredBelow_mkContext_addMotives___spec__1(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withLetDeclImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Meta_IndPredBelow_mkBelow___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__10; static lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkType___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_zip___rarg(lean_object*, lean_object*); @@ -220,14 +222,12 @@ static lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelow LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_IndPredBelow_backwardsChaining___spec__5___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_IndPredBelow_mkContext_addMotives___spec__2(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_forallBoundedTelescope___at_Lean_Meta_arrowDomainsN___spec__6___rarg(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__8; static lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_mkCtorType_mkBelowBinder___spec__3___closed__2; uint64_t lean_uint64_shift_right(uint64_t, uint64_t); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_getBelowIndices(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__3___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__7; lean_object* l_StateRefT_x27_lift___rarg___boxed(lean_object*, lean_object*); lean_object* lean_nat_div(lean_object*, lean_object*); lean_object* l_Lean_MVarId_getType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -242,6 +242,7 @@ lean_object* l_Lean_registerTraceClass(lean_object*, uint8_t, lean_object*, lean static lean_object* l_Lean_Meta_IndPredBelow_mkContext_motiveName___closed__3; LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__3___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_transformFields_loop___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withLocalDeclImp___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -251,7 +252,6 @@ static lean_object* l_Lean_Meta_transform___at_Lean_Meta_IndPredBelow_mkCtorType lean_object* l___private_Lean_CoreM_0__Lean_Core_mkFreshNameImp(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkContext___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__3; static lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow___closed__2; lean_object* l_Lean_mkCasesOn(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_getBelowIndices___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -264,6 +264,7 @@ LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_find lean_object* l_Lean_MVarId_withContext___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_synthPendingImp___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_check(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_closeGoal___closed__8; +static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__1; lean_object* l_Lean_Meta_isInductivePredicate(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__9___rarg(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_FVarId_getDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -272,9 +273,9 @@ lean_object* l_outOfBounds___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkIH___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_applyCtors(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__13; static lean_object* l_Lean_Meta_IndPredBelow_backwardsChaining___lambda__3___closed__1; LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_IndPredBelow_mkBelow___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -288,9 +289,10 @@ static lean_object* l_Lean_Meta_IndPredBelow_mkBelow___closed__1; lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_addBelowPattern___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_append(lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn___closed__2; +static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__2; +static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__5; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkCtorType_replaceTempVars___spec__2(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__2(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__5(lean_object*, lean_object*); @@ -298,17 +300,19 @@ LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Meta_IndPredBelow_m lean_object* l_ST_Prim_Ref_modifyGetUnsafe___rarg___boxed(lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_levelZero; static lean_object* l_Std_Range_forIn_loop___at_Lean_Meta_IndPredBelow_mkBelow___spec__1___closed__2; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_backwardsChaining___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Meta_IndPredBelow_proveBrecOn_applyIH___spec__1(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitLet___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__6___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_replaceTempVars(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_IndPredBelow_mkCtorType_mkBelowBinder___spec__2(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_transform___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__8___boxed(lean_object*, lean_object*); lean_object* l_Lean_Expr_constName_x21(lean_object*); extern lean_object* l_Lean_instInhabitedExpr; -LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142_(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkContext___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MVarId_applyRules(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_constName_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_mkBelowMatcher_transformFields_loop___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -316,31 +320,31 @@ LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_getBelowIndices_loop(lean_obje uint64_t l_Lean_Expr_hash(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkInductiveType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_IndPredBelow_mkContext___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__12; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__3(size_t, size_t, lean_object*); +static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__3; lean_object* l_List_lengthTRAux___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_intros(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_mkCtorType_rebuild___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkContext_mkHeader___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_visit___spec__1(lean_object*, lean_object*); lean_object* l_Lean_Meta_Match_MkMatcherInput_numDiscrs(lean_object*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__1; static lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__3___lambda__5___closed__5; static lean_object* l_Lean_Meta_IndPredBelow_mkBelow___closed__7; uint8_t lean_name_eq(lean_object*, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_applyCtors___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_checkCount___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_lambdaTelescope___at_Lean_PrettyPrinter_Delaborator_returnsPi___spec__1___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_IndPredBelow_mkCtorType_mkBelowBinder___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkType___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_applyIH___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_modifyBinders___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__1(lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__8___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_modifyBinders(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkContext_motiveType___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_checkCount___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_IndPredBelow_backwardsChaining___spec__1(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -360,6 +364,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkIH___lambda__2_ LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkContext_mkHeader(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_getConstInfoInduct___at_Lean_Meta_IndPredBelow_mkContext___spec__1___closed__2; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_applyCtors___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkContext___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_6____closed__3; @@ -367,7 +372,6 @@ lean_object* l_Lean_MessageData_ofExpr(lean_object*); lean_object* l_Lean_throwError___at___private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_checkCount___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_newMotive___lambda__2___closed__2; -static lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__3; uint8_t l_Lean_Expr_binderInfo(lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Meta_IndPredBelow_mkBelow___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_throwError___at_Lean_Meta_mkSimpCongrTheorem___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -396,12 +400,12 @@ LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkContext_motiveName(lean_obje static lean_object* l_Array_forInUnsafe_loop___at_Lean_Meta_IndPredBelow_proveBrecOn_applyIH___spec__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Meta_IndPredBelow_backwardsChaining___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_constLevels_x21(lean_object*); lean_object* l_Lean_Expr_bindingDomain_x21(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__2___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_IndPredBelow_0__Lean_Meta_IndPredBelow_belowType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_instInhabitedVariables___closed__1; +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_addMotives(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Match_Pattern_toMessageData(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkContext(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -411,7 +415,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit___at_Lean_Meta_IndPredBelow LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitLet___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_IndPredBelow_backwardsChaining___spec__5___lambda__2___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_checkCount___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_6____closed__8; lean_object* l_Lean_Expr_app___override(lean_object*, lean_object*); @@ -436,18 +439,16 @@ LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Meta_IndPred static lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_closeGoal___closed__2; lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_backwardsChaining___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__8; +static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__13; static lean_object* l_Lean_Meta_IndPredBelow_mkBrecOnDecl___closed__1; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkContext___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_indentExpr(lean_object*); static lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_IndPredBelow_backwardsChaining___spec__5___lambda__2___closed__5; LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__3___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_Lean_IR_IRType_beq___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getConstInfoInduct___at_Lean_Meta_IndPredBelow_mkContext___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__1; static double l_Lean_addTrace___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__6___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__4; lean_object* l_Lean_Meta_mkForallFVars(lean_object*, lean_object*, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_IndPredBelow_backwardsChaining___spec__5___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_IndPredBelow_mkContext_addMotives___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -460,37 +461,36 @@ LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkIH___lambda__2( LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_findBelowIdx___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_findBelowIdx(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__4; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkContext___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_type(lean_object*); uint64_t lean_uint64_xor(uint64_t, uint64_t); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_addMotives___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_IndPredBelow_mkContext_addMotives___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_indexOfAux___at___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps_visit___spec__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_6____closed__5; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkContext___spec__7___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Array_insertAt_x21___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_closeGoal(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitLambda___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__4___lambda__1(lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_mul(lean_object*, lean_object*); -static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__6; static lean_object* l_Lean_getConstInfoInduct___at_Lean_Meta_IndPredBelow_mkContext___spec__1___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__11(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_mkCtorType_mkBelowBinder___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__1; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_closeGoal___closed__6; lean_object* l_Lean_mkArrow(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_visit___spec__2(lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_mkBelow___closed__5; static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__16___rarg___closed__6; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkContext___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_ofSubarray___rarg(lean_object*); lean_object* l_Lean_MVarId_apply(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_IndPredBelow_backwardsChaining___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_back___rarg(lean_object*, lean_object*); lean_object* lean_expr_instantiate_rev(lean_object*, lean_object*); @@ -498,24 +498,25 @@ LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_copyVarName(lean_ob lean_object* l_List_reverse___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_backwardsChaining___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__16___rarg___closed__4; +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__3; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_applyCtors___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Meta_IndPredBelow_backwardsChaining___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_IndPredBelow_mkCtorType_mkBelowBinder___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_sub(size_t, size_t); lean_object* lean_array_mk(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_IndPredBelow_mkBelow___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_lambdaTelescope___at_Lean_PrettyPrinter_Delaborator_returnsPi___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_6____closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_introNPRec(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkContext___spec__6(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__6; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkCtorType_replaceTempVars___spec__1(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_closeGoal___closed__9; extern lean_object* l_Lean_instInhabitedName; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__12; lean_object* lean_array_uget(lean_object*, size_t); lean_object* l_Lean_Expr_fvar___override(lean_object*); size_t lean_array_size(lean_object*); @@ -536,36 +537,31 @@ static lean_object* l_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkIH___closed__3; LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__3___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_addBelowPattern(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__3___lambda__5___closed__3; -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__3(lean_object*); lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkContext_motiveType___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_IndPredBelow_mkCtorType_mkBelowBinder___spec__1(lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_backwardsChaining___lambda__3___closed__5; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__2; -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Meta_IndPredBelow_backwardsChaining___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_newMotive___lambda__1___closed__2; static lean_object* l_Lean_Meta_transform___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_newMotive___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__3___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_mkMotiveBinder___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_string_append(lean_object*, lean_object*); lean_object* l_Lean_isTracingEnabledFor___at_Lean_Meta_processPostponed_loop___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkFreshExprSyntheticOpaqueMVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__10; LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__9___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); lean_object* l_Lean_LocalDecl_toExpr(lean_object*); LEAN_EXPORT uint8_t l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_mkCtorType_mkBelowBinder___spec__3___lambda__1(lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_loop___at_Lean_Meta_IndPredBelow_mkBelow___spec__1___closed__3; -static lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__2; +static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__11; static lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_mkCtorType_mkBelowBinder___spec__3___closed__1; lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowDecl___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkContext___spec__3(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_IndPredBelow_proveBrecOn_applyCtors___spec__4(lean_object*, size_t, size_t, lean_object*); @@ -573,9 +569,7 @@ lean_object* l_List_mapTR_loop___at_Lean_Meta_Match_Alt_toMessageData___spec__2( lean_object* l_Lean_Meta_intro1Core(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_closeGoal___closed__4; lean_object* l_Lean_Meta_mkLambdaFVars(lean_object*, lean_object*, uint8_t, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkType___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow___lambda__3___closed__1; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_applyCtors___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); static lean_object* l_Lean_Meta_transform_visit___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__2___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkContext_addMotives___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -591,13 +585,14 @@ LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitPost___at_Lean_Meta_In uint8_t l_Lean_Exception_isRuntime(lean_object*); static lean_object* l_Lean_Meta_transform___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__1___closed__3; static lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_closeGoal___closed__5; -static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__11; uint8_t l_Lean_Expr_isForall(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_checkCount___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_mvarId_x21(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_addBelowPattern___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144_(lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_checkCount___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_transform___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Meta_Match_instInhabitedPattern; @@ -622,9 +617,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow_ static lean_object* l_Std_Range_forIn_loop___at_Lean_Meta_IndPredBelow_mkBelow___spec__1___closed__4; static lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_transformFields_loop___closed__2; lean_object* l_Lean_Meta_withNewBinderInfos___at_Lean_Meta_withInstImplicitAsImplict___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_intros___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkContext___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__3___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__7___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_mkBelowBinder(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1712,7 +1705,7 @@ return x_24; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkContext___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkContext___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { lean_object* x_12; uint8_t x_13; @@ -1943,7 +1936,7 @@ lean_dec(x_18); x_21 = lean_array_get_size(x_19); x_22 = lean_mk_empty_array_with_capacity(x_21); x_23 = lean_unsigned_to_nat(0u); -x_24 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkContext___spec__5(x_19, x_19, x_21, x_23, lean_box(0), x_22, x_2, x_3, x_4, x_5, x_20); +x_24 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkContext___spec__5(x_19, x_19, x_21, x_23, lean_box(0), x_22, x_2, x_3, x_4, x_5, x_20); lean_dec(x_19); x_25 = lean_ctor_get(x_24, 0); lean_inc(x_25); @@ -2161,11 +2154,11 @@ x_11 = l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkContext___spec__4(x_ return x_11; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkContext___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkContext___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { lean_object* x_12; -x_12 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkContext___spec__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_12 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkContext___spec__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -10018,132 +10011,6 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__3___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; lean_object* x_12; -x_11 = lean_array_push(x_1, x_5); -x_12 = l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__3___rarg(x_2, x_3, x_4, x_11, x_6, x_7, x_8, x_9, x_10); -return x_12; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_10 = lean_array_get_size(x_4); -x_11 = lean_array_get_size(x_1); -x_12 = lean_nat_dec_lt(x_10, x_11); -lean_dec(x_11); -if (x_12 == 0) -{ -lean_object* x_13; -lean_dec(x_10); -lean_dec(x_3); -lean_dec(x_1); -x_13 = lean_apply_6(x_2, x_4, x_5, x_6, x_7, x_8, x_9); -return x_13; -} -else -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_14 = lean_array_fget(x_1, x_10); -lean_dec(x_10); -x_15 = lean_ctor_get(x_14, 1); -lean_inc(x_15); -x_16 = lean_ctor_get(x_14, 0); -lean_inc(x_16); -lean_dec(x_14); -x_17 = lean_ctor_get(x_15, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_15, 1); -lean_inc(x_18); -lean_dec(x_15); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -x_19 = lean_apply_6(x_18, x_4, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_19) == 0) -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; uint8_t x_24; lean_object* x_25; -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_19, 1); -lean_inc(x_21); -lean_dec(x_19); -x_22 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__3___rarg___lambda__1), 10, 4); -lean_closure_set(x_22, 0, x_4); -lean_closure_set(x_22, 1, x_1); -lean_closure_set(x_22, 2, x_2); -lean_closure_set(x_22, 3, x_3); -x_23 = 0; -x_24 = lean_unbox(x_17); -lean_dec(x_17); -x_25 = l_Lean_Meta_withLocalDecl___at_Lean_Meta_GeneralizeTelescope_generalizeTelescopeAux___spec__1___rarg(x_16, x_24, x_20, x_22, x_23, x_5, x_6, x_7, x_8, x_21); -return x_25; -} -else -{ -uint8_t x_26; -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_26 = !lean_is_exclusive(x_19); -if (x_26 == 0) -{ -return x_19; -} -else -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_19, 0); -x_28 = lean_ctor_get(x_19, 1); -lean_inc(x_28); -lean_inc(x_27); -lean_dec(x_19); -x_29 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_29, 0, x_27); -lean_ctor_set(x_29, 1, x_28); -return x_29; -} -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__3(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__3___rarg), 9, 0); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; lean_object* x_10; -x_9 = l_Lean_Meta_transform_visit___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__2___lambda__1___closed__1; -x_10 = l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__3___rarg(x_2, x_3, x_1, x_9, x_4, x_5, x_6, x_7, x_8); -return x_10; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__2(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecls___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__2___rarg), 8, 0); -return x_2; -} -} LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_addMotives___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { @@ -10211,7 +10078,7 @@ lean_closure_set(x_16, 1, x_1); lean_closure_set(x_16, 2, x_2); lean_closure_set(x_16, 3, x_3); x_17 = l_Lean_instInhabitedExpr; -x_18 = l_Lean_Meta_withLocalDecls___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__2___rarg(x_17, x_14, x_16, x_5, x_6, x_7, x_8, x_15); +x_18 = l_Lean_Meta_withLocalDecls___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__4___rarg(x_17, x_14, x_16, x_5, x_6, x_7, x_8, x_15); return x_18; } } @@ -10241,7 +10108,7 @@ lean_dec(x_5); return x_12; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; @@ -10251,145 +10118,69 @@ lean_ctor_set(x_8, 1, x_7); return x_8; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_12; uint8_t x_13; -x_12 = lean_unsigned_to_nat(0u); -x_13 = lean_nat_dec_eq(x_3, x_12); -if (x_13 == 0) -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; -x_14 = lean_unsigned_to_nat(1u); -x_15 = lean_nat_sub(x_3, x_14); -lean_dec(x_3); -x_16 = lean_array_fget(x_2, x_4); -x_17 = lean_ctor_get(x_1, 2); -x_18 = lean_array_get_size(x_17); -x_19 = lean_nat_dec_lt(x_4, x_18); -lean_dec(x_18); -x_20 = lean_alloc_closure((void*)(l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__1___lambda__1___boxed), 7, 1); -lean_closure_set(x_20, 0, x_16); -if (x_19 == 0) -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_21 = l_Lean_instInhabitedName; -x_22 = l_outOfBounds___rarg(x_21); -x_23 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_23, 0, x_22); -lean_ctor_set(x_23, 1, x_20); -x_24 = lean_nat_add(x_4, x_14); -lean_dec(x_4); -x_25 = lean_array_push(x_6, x_23); -x_3 = x_15; -x_4 = x_24; -x_5 = lean_box(0); -x_6 = x_25; -goto _start; -} -else -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_27 = lean_array_fget(x_17, x_4); -x_28 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_28, 0, x_27); -lean_ctor_set(x_28, 1, x_20); -x_29 = lean_nat_add(x_4, x_14); -lean_dec(x_4); -x_30 = lean_array_push(x_6, x_28); -x_3 = x_15; -x_4 = x_29; -x_5 = lean_box(0); -x_6 = x_30; -goto _start; -} -} -else +lean_object* x_13; uint8_t x_14; +x_13 = lean_unsigned_to_nat(0u); +x_14 = lean_nat_dec_eq(x_4, x_13); +if (x_14 == 0) { -lean_object* x_32; +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; lean_object* x_21; +x_15 = lean_unsigned_to_nat(1u); +x_16 = lean_nat_sub(x_4, x_15); lean_dec(x_4); -lean_dec(x_3); -x_32 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_32, 0, x_6); -lean_ctor_set(x_32, 1, x_11); -return x_32; -} -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__3(size_t x_1, size_t x_2, lean_object* x_3) { -_start: -{ -uint8_t x_4; -x_4 = lean_usize_dec_lt(x_2, x_1); -if (x_4 == 0) -{ -return x_3; -} -else -{ -lean_object* x_5; lean_object* x_6; lean_object* x_7; size_t x_8; size_t x_9; uint8_t x_10; -x_5 = lean_array_uget(x_3, x_2); -x_6 = lean_unsigned_to_nat(0u); -x_7 = lean_array_uset(x_3, x_2, x_6); -x_8 = 1; -x_9 = lean_usize_add(x_2, x_8); -x_10 = !lean_is_exclusive(x_5); -if (x_10 == 0) +x_17 = lean_array_fget(x_3, x_5); +x_18 = lean_ctor_get(x_1, 2); +x_19 = lean_array_get_size(x_18); +x_20 = lean_nat_dec_lt(x_5, x_19); +lean_dec(x_19); +x_21 = lean_alloc_closure((void*)(l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__1___lambda__1___boxed), 7, 1); +lean_closure_set(x_21, 0, x_17); +if (x_20 == 0) { -lean_object* x_11; uint8_t x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_11 = lean_ctor_get(x_5, 0); -x_12 = 0; -x_13 = lean_box(x_12); -lean_ctor_set(x_5, 0, x_13); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_11); -lean_ctor_set(x_14, 1, x_5); -x_15 = lean_array_uset(x_7, x_2, x_14); -x_2 = x_9; -x_3 = x_15; +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_22 = l_Lean_instInhabitedName; +x_23 = l_outOfBounds___rarg(x_22); +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_23); +lean_ctor_set(x_24, 1, x_21); +x_25 = lean_nat_add(x_5, x_15); +lean_dec(x_5); +x_26 = lean_array_push(x_7, x_24); +x_4 = x_16; +x_5 = x_25; +x_6 = lean_box(0); +x_7 = x_26; goto _start; } else { -lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_17 = lean_ctor_get(x_5, 0); -x_18 = lean_ctor_get(x_5, 1); -lean_inc(x_18); -lean_inc(x_17); +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_28 = lean_array_fget(x_18, x_5); +x_29 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_21); +x_30 = lean_nat_add(x_5, x_15); lean_dec(x_5); -x_19 = 0; -x_20 = lean_box(x_19); -x_21 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_21, 0, x_20); -lean_ctor_set(x_21, 1, x_18); -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_17); -lean_ctor_set(x_22, 1, x_21); -x_23 = lean_array_uset(x_7, x_2, x_22); -x_2 = x_9; -x_3 = x_23; +x_31 = lean_array_push(x_7, x_29); +x_4 = x_16; +x_5 = x_30; +x_6 = lean_box(0); +x_7 = x_31; goto _start; } } -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: +else { -size_t x_9; size_t x_10; lean_object* x_11; lean_object* x_12; -x_9 = lean_array_size(x_2); -x_10 = 0; -x_11 = l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__3(x_9, x_10, x_2); -x_12 = l_Lean_Meta_withLocalDecls___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__2___rarg(x_1, x_11, x_3, x_4, x_5, x_6, x_7, x_8); -return x_12; -} +lean_object* x_33; +lean_dec(x_5); +lean_dec(x_4); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_7); +lean_ctor_set(x_33, 1, x_12); +return x_33; } -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__2(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__2___rarg), 8, 0); -return x_2; } } LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { @@ -10441,7 +10232,7 @@ lean_inc(x_10); x_11 = lean_array_get_size(x_10); x_12 = lean_mk_empty_array_with_capacity(x_11); x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__1(x_1, x_10, x_11, x_13, lean_box(0), x_12, x_5, x_6, x_7, x_8, x_9); +x_14 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__1(x_1, x_10, x_10, x_11, x_13, lean_box(0), x_12, x_5, x_6, x_7, x_8, x_9); lean_dec(x_10); x_15 = lean_ctor_get(x_14, 0); lean_inc(x_15); @@ -10454,15 +10245,15 @@ lean_closure_set(x_17, 1, x_1); lean_closure_set(x_17, 2, x_2); lean_closure_set(x_17, 3, x_3); x_18 = l_Lean_instInhabitedExpr; -x_19 = l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__2___rarg(x_18, x_15, x_17, x_5, x_6, x_7, x_8, x_16); +x_19 = l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__2___rarg(x_18, x_15, x_17, x_5, x_6, x_7, x_8, x_16); return x_19; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; -x_8 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); @@ -10471,30 +10262,19 @@ lean_dec(x_2); return x_8; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_12; -x_12 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_object* x_13; +x_13 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_7); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -return x_12; -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -size_t x_4; size_t x_5; lean_object* x_6; -x_4 = lean_unbox_usize(x_1); -lean_dec(x_1); -x_5 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_6 = l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__3(x_4, x_5, x_3); -return x_6; +return x_13; } } LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { @@ -11102,89 +10882,89 @@ return x_61; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowDecl___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowDecl___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_12; uint8_t x_13; -x_12 = lean_unsigned_to_nat(0u); -x_13 = lean_nat_dec_eq(x_3, x_12); -if (x_13 == 0) +lean_object* x_13; uint8_t x_14; +x_13 = lean_unsigned_to_nat(0u); +x_14 = lean_nat_dec_eq(x_4, x_13); +if (x_14 == 0) { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_14 = lean_unsigned_to_nat(1u); -x_15 = lean_nat_sub(x_3, x_14); -lean_dec(x_3); -x_16 = lean_array_fget(x_2, x_4); +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_15 = lean_unsigned_to_nat(1u); +x_16 = lean_nat_sub(x_4, x_15); +lean_dec(x_4); +x_17 = lean_array_fget(x_3, x_5); +lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_4); +lean_inc(x_5); lean_inc(x_1); -x_17 = l_Lean_Meta_IndPredBelow_mkInductiveType(x_1, x_4, x_16, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_17) == 0) +x_18 = l_Lean_Meta_IndPredBelow_mkInductiveType(x_1, x_5, x_17, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_18) == 0) { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_17, 1); +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_19 = lean_ctor_get(x_18, 0); lean_inc(x_19); -lean_dec(x_17); -x_20 = lean_nat_add(x_4, x_14); -lean_dec(x_4); -x_21 = lean_array_push(x_6, x_18); -x_3 = x_15; -x_4 = x_20; -x_5 = lean_box(0); -x_6 = x_21; -x_11 = x_19; +x_20 = lean_ctor_get(x_18, 1); +lean_inc(x_20); +lean_dec(x_18); +x_21 = lean_nat_add(x_5, x_15); +lean_dec(x_5); +x_22 = lean_array_push(x_7, x_19); +x_4 = x_16; +x_5 = x_21; +x_6 = lean_box(0); +x_7 = x_22; +x_12 = x_20; goto _start; } else { -uint8_t x_23; -lean_dec(x_15); +uint8_t x_24; +lean_dec(x_16); +lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_4); +lean_dec(x_5); lean_dec(x_1); -x_23 = !lean_is_exclusive(x_17); -if (x_23 == 0) +x_24 = !lean_is_exclusive(x_18); +if (x_24 == 0) { -return x_17; +return x_18; } else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_17, 0); -x_25 = lean_ctor_get(x_17, 1); +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_18, 0); +x_26 = lean_ctor_get(x_18, 1); +lean_inc(x_26); lean_inc(x_25); -lean_inc(x_24); -lean_dec(x_17); -x_26 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_26, 0, x_24); -lean_ctor_set(x_26, 1, x_25); -return x_26; +lean_dec(x_18); +x_27 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +return x_27; } } } else { -lean_object* x_27; +lean_object* x_28; +lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_7); +lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); lean_dec(x_1); -x_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_6); -lean_ctor_set(x_27, 1, x_11); -return x_27; +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_7); +lean_ctor_set(x_28, 1, x_12); +return x_28; } } } @@ -11199,7 +10979,7 @@ x_9 = lean_unsigned_to_nat(0u); x_10 = lean_nat_dec_lt(x_9, x_8); x_11 = lean_mk_empty_array_with_capacity(x_8); lean_inc(x_1); -x_12 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowDecl___spec__1(x_1, x_7, x_8, x_9, lean_box(0), x_11, x_2, x_3, x_4, x_5, x_6); +x_12 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowDecl___spec__1(x_1, x_7, x_7, x_8, x_9, lean_box(0), x_11, x_2, x_3, x_4, x_5, x_6); if (x_10 == 0) { lean_dec(x_7); @@ -11406,13 +11186,14 @@ return x_72; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowDecl___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowDecl___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_12; -x_12 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowDecl___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_object* x_13; +x_13 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowDecl___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_3); lean_dec(x_2); -return x_12; +return x_13; } } LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_IndPredBelow_backwardsChaining___spec__1(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { @@ -14381,7 +14162,7 @@ lean_dec(x_2); return x_8; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; uint8_t x_15; lean_object* x_16; lean_object* x_17; @@ -14420,155 +14201,155 @@ return x_32; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { -lean_object* x_15; uint8_t x_16; -x_15 = lean_unsigned_to_nat(0u); -x_16 = lean_nat_dec_eq(x_6, x_15); -if (x_16 == 0) +lean_object* x_16; uint8_t x_17; +x_16 = lean_unsigned_to_nat(0u); +x_17 = lean_nat_dec_eq(x_7, x_16); +if (x_17 == 0) { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_17 = lean_unsigned_to_nat(1u); -x_18 = lean_nat_sub(x_6, x_17); -lean_dec(x_6); -x_19 = lean_array_fget(x_5, x_7); -x_20 = lean_ctor_get(x_19, 1); -lean_inc(x_20); -lean_dec(x_19); +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_18 = lean_unsigned_to_nat(1u); +x_19 = lean_nat_sub(x_7, x_18); +lean_dec(x_7); +x_20 = lean_array_fget(x_6, x_8); +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); -lean_inc(x_10); -x_21 = l___private_Lean_Meta_Basic_0__Lean_Meta_instantiateForallAux(x_2, x_15, x_20, x_10, x_11, x_12, x_13, x_14); -if (lean_obj_tag(x_21) == 0) +x_22 = l___private_Lean_Meta_Basic_0__Lean_Meta_instantiateForallAux(x_2, x_16, x_21, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_22) == 0) { -lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; lean_object* x_26; -x_22 = lean_ctor_get(x_21, 0); -lean_inc(x_22); -x_23 = lean_ctor_get(x_21, 1); +lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; lean_object* x_27; +x_23 = lean_ctor_get(x_22, 0); lean_inc(x_23); -lean_dec(x_21); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +lean_dec(x_22); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); -lean_inc(x_7); +lean_inc(x_8); lean_inc(x_1); -x_24 = lean_alloc_closure((void*)(l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___spec__1___lambda__1___boxed), 12, 5); -lean_closure_set(x_24, 0, x_1); -lean_closure_set(x_24, 1, x_7); -lean_closure_set(x_24, 2, x_2); -lean_closure_set(x_24, 3, x_3); -lean_closure_set(x_24, 4, x_4); -x_25 = 0; +x_25 = lean_alloc_closure((void*)(l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___spec__1___lambda__1___boxed), 12, 5); +lean_closure_set(x_25, 0, x_1); +lean_closure_set(x_25, 1, x_8); +lean_closure_set(x_25, 2, x_2); +lean_closure_set(x_25, 3, x_3); +lean_closure_set(x_25, 4, x_4); +x_26 = 0; +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); -lean_inc(x_10); -x_26 = l_Lean_Meta_forallTelescopeReducing___at_Lean_Meta_getParamNames___spec__2___rarg(x_22, x_24, x_25, x_10, x_11, x_12, x_13, x_23); -if (lean_obj_tag(x_26) == 0) +x_27 = l_Lean_Meta_forallTelescopeReducing___at_Lean_Meta_getParamNames___spec__2___rarg(x_23, x_25, x_26, x_11, x_12, x_13, x_14, x_24); +if (lean_obj_tag(x_27) == 0) { -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_27 = lean_ctor_get(x_26, 0); -lean_inc(x_27); -x_28 = lean_ctor_get(x_26, 1); +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_28 = lean_ctor_get(x_27, 0); lean_inc(x_28); -lean_dec(x_26); -x_29 = lean_nat_add(x_7, x_17); -lean_dec(x_7); -x_30 = lean_array_push(x_9, x_27); -x_6 = x_18; -x_7 = x_29; -x_8 = lean_box(0); -x_9 = x_30; -x_14 = x_28; +x_29 = lean_ctor_get(x_27, 1); +lean_inc(x_29); +lean_dec(x_27); +x_30 = lean_nat_add(x_8, x_18); +lean_dec(x_8); +x_31 = lean_array_push(x_10, x_28); +x_7 = x_19; +x_8 = x_30; +x_9 = lean_box(0); +x_10 = x_31; +x_15 = x_29; goto _start; } else { -uint8_t x_32; -lean_dec(x_18); +uint8_t x_33; +lean_dec(x_19); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_7); +lean_dec(x_8); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_32 = !lean_is_exclusive(x_26); -if (x_32 == 0) +x_33 = !lean_is_exclusive(x_27); +if (x_33 == 0) { -return x_26; +return x_27; } else { -lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_33 = lean_ctor_get(x_26, 0); -x_34 = lean_ctor_get(x_26, 1); +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_27, 0); +x_35 = lean_ctor_get(x_27, 1); +lean_inc(x_35); lean_inc(x_34); -lean_inc(x_33); -lean_dec(x_26); -x_35 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_35, 0, x_33); -lean_ctor_set(x_35, 1, x_34); -return x_35; +lean_dec(x_27); +x_36 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_36, 0, x_34); +lean_ctor_set(x_36, 1, x_35); +return x_36; } } } else { -uint8_t x_36; -lean_dec(x_18); +uint8_t x_37; +lean_dec(x_19); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_7); +lean_dec(x_8); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_36 = !lean_is_exclusive(x_21); -if (x_36 == 0) +x_37 = !lean_is_exclusive(x_22); +if (x_37 == 0) { -return x_21; +return x_22; } else { -lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_37 = lean_ctor_get(x_21, 0); -x_38 = lean_ctor_get(x_21, 1); +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_22, 0); +x_39 = lean_ctor_get(x_22, 1); +lean_inc(x_39); lean_inc(x_38); -lean_inc(x_37); -lean_dec(x_21); -x_39 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_39, 0, x_37); -lean_ctor_set(x_39, 1, x_38); -return x_39; +lean_dec(x_22); +x_40 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +return x_40; } } } else { -lean_object* x_40; +lean_object* x_41; +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); -lean_dec(x_10); +lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_40 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_40, 0, x_9); -lean_ctor_set(x_40, 1, x_14); -return x_40; +x_41 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_41, 0, x_10); +lean_ctor_set(x_41, 1, x_15); +return x_41; } } } @@ -14612,7 +14393,7 @@ lean_inc(x_6); lean_inc(x_5); lean_inc(x_20); lean_inc(x_13); -x_25 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___spec__1(x_1, x_13, x_16, x_20, x_21, x_22, x_24, lean_box(0), x_23, x_5, x_6, x_7, x_8, x_9); +x_25 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___spec__1(x_1, x_13, x_16, x_20, x_21, x_21, x_22, x_24, lean_box(0), x_23, x_5, x_6, x_7, x_8, x_9); lean_dec(x_21); if (lean_obj_tag(x_25) == 0) { @@ -14733,11 +14514,11 @@ return x_56; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; -x_13 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_13 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -14749,13 +14530,14 @@ lean_dec(x_1); return x_13; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { -lean_object* x_15; -x_15 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_object* x_16; +x_16 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +lean_dec(x_6); lean_dec(x_5); -return x_15; +return x_16; } } LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_introNPRec(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { @@ -15120,7 +14902,7 @@ return x_25; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_applyCtors___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_applyCtors___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { lean_object* x_12; uint8_t x_13; @@ -15318,14 +15100,12 @@ LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_applyCtors(lean_ob _start: { lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; -lean_inc(x_1); x_7 = lean_array_mk(x_1); x_8 = lean_array_get_size(x_7); x_9 = lean_mk_empty_array_with_capacity(x_8); x_10 = lean_unsigned_to_nat(0u); -x_11 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_applyCtors___spec__3(x_1, x_7, x_8, x_10, lean_box(0), x_9, x_2, x_3, x_4, x_5, x_6); +x_11 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_applyCtors___spec__3(x_7, x_7, x_8, x_10, lean_box(0), x_9, x_2, x_3, x_4, x_5, x_6); lean_dec(x_7); -lean_dec(x_1); if (lean_obj_tag(x_11) == 0) { uint8_t x_12; @@ -15425,11 +15205,11 @@ lean_dec(x_2); return x_11; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_applyCtors___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_applyCtors___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { lean_object* x_12; -x_12 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_applyCtors___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_12 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_applyCtors___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_2); lean_dec(x_1); return x_12; @@ -16461,95 +16241,95 @@ lean_dec(x_6); return x_12; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkType___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkType___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { -lean_object* x_14; uint8_t x_15; -x_14 = lean_unsigned_to_nat(0u); -x_15 = lean_nat_dec_eq(x_5, x_14); -if (x_15 == 0) +lean_object* x_15; uint8_t x_16; +x_15 = lean_unsigned_to_nat(0u); +x_16 = lean_nat_dec_eq(x_6, x_15); +if (x_16 == 0) { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_16 = lean_unsigned_to_nat(1u); -x_17 = lean_nat_sub(x_5, x_16); -lean_dec(x_5); -x_18 = lean_array_fget(x_4, x_6); +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_17 = lean_unsigned_to_nat(1u); +x_18 = lean_nat_sub(x_6, x_17); +lean_dec(x_6); +x_19 = lean_array_fget(x_5, x_7); +lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_6); -lean_inc(x_2); +lean_inc(x_7); lean_inc(x_3); +lean_inc(x_4); lean_inc(x_1); -x_19 = l_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkIH(x_1, x_3, x_2, x_6, x_18, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_19) == 0) +x_20 = l_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkIH(x_1, x_4, x_3, x_7, x_19, x_10, x_11, x_12, x_13, x_14); +if (lean_obj_tag(x_20) == 0) { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_19, 1); +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_21 = lean_ctor_get(x_20, 0); lean_inc(x_21); -lean_dec(x_19); -x_22 = lean_nat_add(x_6, x_16); -lean_dec(x_6); -x_23 = lean_array_push(x_8, x_20); -x_5 = x_17; -x_6 = x_22; -x_7 = lean_box(0); -x_8 = x_23; -x_13 = x_21; +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +x_23 = lean_nat_add(x_7, x_17); +lean_dec(x_7); +x_24 = lean_array_push(x_9, x_21); +x_6 = x_18; +x_7 = x_23; +x_8 = lean_box(0); +x_9 = x_24; +x_14 = x_22; goto _start; } else { -uint8_t x_25; -lean_dec(x_17); +uint8_t x_26; +lean_dec(x_18); +lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_6); +lean_dec(x_7); +lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); lean_dec(x_1); -x_25 = !lean_is_exclusive(x_19); -if (x_25 == 0) +x_26 = !lean_is_exclusive(x_20); +if (x_26 == 0) { -return x_19; +return x_20; } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_19, 0); -x_27 = lean_ctor_get(x_19, 1); +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_20, 0); +x_28 = lean_ctor_get(x_20, 1); +lean_inc(x_28); lean_inc(x_27); -lean_inc(x_26); -lean_dec(x_19); -x_28 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_28, 0, x_26); -lean_ctor_set(x_28, 1, x_27); -return x_28; +lean_dec(x_20); +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_27); +lean_ctor_set(x_29, 1, x_28); +return x_29; } } } else { -lean_object* x_29; +lean_object* x_30; +lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); -lean_dec(x_9); +lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); lean_dec(x_1); -x_29 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_29, 0, x_8); -lean_ctor_set(x_29, 1, x_13); -return x_29; +x_30 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_30, 0, x_9); +lean_ctor_set(x_30, 1, x_14); +return x_30; } } } @@ -16619,7 +16399,7 @@ lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_17); -x_22 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkType___spec__1(x_1, x_17, x_20, x_13, x_14, x_11, lean_box(0), x_21, x_5, x_6, x_7, x_8, x_9); +x_22 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkType___spec__1(x_1, x_13, x_17, x_20, x_13, x_14, x_11, lean_box(0), x_21, x_5, x_6, x_7, x_8, x_9); lean_dec(x_13); if (lean_obj_tag(x_22) == 0) { @@ -16635,7 +16415,7 @@ lean_closure_set(x_25, 1, x_17); lean_closure_set(x_25, 2, x_2); lean_closure_set(x_25, 3, x_19); x_26 = l_Lean_instInhabitedExpr; -x_27 = l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__2___rarg(x_26, x_23, x_25, x_5, x_6, x_7, x_8, x_24); +x_27 = l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__2___rarg(x_26, x_23, x_25, x_5, x_6, x_7, x_8, x_24); return x_27; } else @@ -16706,13 +16486,14 @@ return x_18; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkType___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkType___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { -lean_object* x_14; -x_14 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkType___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_4); -return x_14; +lean_object* x_15; +x_15 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkType___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_5); +lean_dec(x_2); +return x_15; } } LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkType___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { @@ -20282,7 +20063,7 @@ goto _start; } } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__1() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__1() { _start: { lean_object* x_1; @@ -20290,16 +20071,16 @@ x_1 = lean_mk_string_unchecked("alt ", 4, 4); return x_1; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__2() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__1; +x_1 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__3() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__3() { _start: { lean_object* x_1; @@ -20307,16 +20088,16 @@ x_1 = lean_mk_string_unchecked(":\n", 2, 2); return x_1; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__4() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__3; +x_1 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__3; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; uint8_t x_24; uint8_t x_25; lean_object* x_26; @@ -20388,11 +20169,11 @@ x_37 = l___private_Init_Data_Repr_0__Nat_reprFast(x_7); x_38 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_38, 0, x_37); x_39 = l_Lean_MessageData_ofFormat(x_38); -x_40 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__2; +x_40 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__2; x_41 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_41, 0, x_40); lean_ctor_set(x_41, 1, x_39); -x_42 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__4; +x_42 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__4; x_43 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_43, 0, x_41); lean_ctor_set(x_43, 1, x_42); @@ -20463,7 +20244,7 @@ return x_60; } } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__1() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__1() { _start: { lean_object* x_1; @@ -20471,16 +20252,16 @@ x_1 = lean_mk_string_unchecked("xs = ", 5, 5); return x_1; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__2() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__1; +x_1 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__3() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__3() { _start: { lean_object* x_1; @@ -20488,16 +20269,16 @@ x_1 = lean_mk_string_unchecked("; oldFVars = ", 13, 13); return x_1; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__4() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__3; +x_1 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__3; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__5() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__5() { _start: { lean_object* x_1; @@ -20505,16 +20286,16 @@ x_1 = lean_mk_string_unchecked("; fvars = ", 10, 10); return x_1; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__6() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__6() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__5; +x_1 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__5; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__7() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__7() { _start: { lean_object* x_1; @@ -20522,16 +20303,16 @@ x_1 = lean_mk_string_unchecked("; new = ", 8, 8); return x_1; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__8() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__8() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__7; +x_1 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__7; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { lean_object* x_12; lean_object* x_13; size_t x_14; size_t x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; @@ -20603,7 +20384,7 @@ lean_object* x_33; lean_object* x_34; lean_free_object(x_24); lean_dec(x_12); x_33 = lean_box(0); -x_34 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1(x_25, x_17, x_22, x_16, x_31, x_23, x_3, x_4, x_33, x_7, x_8, x_9, x_10, x_28); +x_34 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1(x_25, x_17, x_22, x_16, x_31, x_23, x_3, x_4, x_33, x_7, x_8, x_9, x_10, x_28); return x_34; } else @@ -20614,11 +20395,11 @@ x_35 = lean_array_to_list(x_25); x_36 = lean_box(0); x_37 = l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(x_35, x_36); x_38 = l_Lean_MessageData_ofList(x_37); -x_39 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__2; +x_39 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__2; lean_ctor_set_tag(x_24, 7); lean_ctor_set(x_24, 1, x_38); lean_ctor_set(x_24, 0, x_39); -x_40 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__4; +x_40 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__4; x_41 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_41, 0, x_24); lean_ctor_set(x_41, 1, x_40); @@ -20630,7 +20411,7 @@ x_46 = l_Lean_MessageData_ofList(x_45); x_47 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_47, 0, x_41); lean_ctor_set(x_47, 1, x_46); -x_48 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__6; +x_48 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__6; x_49 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_49, 0, x_47); lean_ctor_set(x_49, 1, x_48); @@ -20641,7 +20422,7 @@ x_52 = l_Lean_MessageData_ofList(x_51); x_53 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_53, 0, x_49); lean_ctor_set(x_53, 1, x_52); -x_54 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__8; +x_54 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__8; x_55 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_55, 0, x_53); lean_ctor_set(x_55, 1, x_54); @@ -20686,7 +20467,7 @@ lean_inc(x_77); x_78 = lean_ctor_get(x_76, 1); lean_inc(x_78); lean_dec(x_76); -x_79 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1(x_25, x_17, x_22, x_16, x_31, x_23, x_3, x_4, x_77, x_7, x_8, x_9, x_10, x_78); +x_79 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1(x_25, x_17, x_22, x_16, x_31, x_23, x_3, x_4, x_77, x_7, x_8, x_9, x_10, x_78); lean_dec(x_77); return x_79; } @@ -20713,7 +20494,7 @@ if (x_85 == 0) lean_object* x_86; lean_object* x_87; lean_dec(x_12); x_86 = lean_box(0); -x_87 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1(x_25, x_17, x_22, x_16, x_84, x_23, x_3, x_4, x_86, x_7, x_8, x_9, x_10, x_81); +x_87 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1(x_25, x_17, x_22, x_16, x_84, x_23, x_3, x_4, x_86, x_7, x_8, x_9, x_10, x_81); return x_87; } else @@ -20724,11 +20505,11 @@ x_88 = lean_array_to_list(x_25); x_89 = lean_box(0); x_90 = l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(x_88, x_89); x_91 = l_Lean_MessageData_ofList(x_90); -x_92 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__2; +x_92 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__2; x_93 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_93, 0, x_92); lean_ctor_set(x_93, 1, x_91); -x_94 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__4; +x_94 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__4; x_95 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_95, 0, x_93); lean_ctor_set(x_95, 1, x_94); @@ -20740,7 +20521,7 @@ x_100 = l_Lean_MessageData_ofList(x_99); x_101 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_101, 0, x_95); lean_ctor_set(x_101, 1, x_100); -x_102 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__6; +x_102 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__6; x_103 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_103, 0, x_101); lean_ctor_set(x_103, 1, x_102); @@ -20751,7 +20532,7 @@ x_106 = l_Lean_MessageData_ofList(x_105); x_107 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_107, 0, x_103); lean_ctor_set(x_107, 1, x_106); -x_108 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__8; +x_108 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__8; x_109 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_109, 0, x_107); lean_ctor_set(x_109, 1, x_108); @@ -20796,7 +20577,7 @@ lean_inc(x_131); x_132 = lean_ctor_get(x_130, 1); lean_inc(x_132); lean_dec(x_130); -x_133 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1(x_25, x_17, x_22, x_16, x_84, x_23, x_3, x_4, x_131, x_7, x_8, x_9, x_10, x_132); +x_133 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1(x_25, x_17, x_22, x_16, x_84, x_23, x_3, x_4, x_131, x_7, x_8, x_9, x_10, x_132); lean_dec(x_131); return x_133; } @@ -20804,117 +20585,117 @@ return x_133; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_14; uint8_t x_15; -x_14 = lean_unsigned_to_nat(0u); -x_15 = lean_nat_dec_eq(x_5, x_14); -if (x_15 == 0) +lean_object* x_12; uint8_t x_13; +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_nat_dec_eq(x_3, x_12); +if (x_13 == 0) { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_16 = lean_unsigned_to_nat(1u); -x_17 = lean_nat_sub(x_5, x_16); -lean_dec(x_5); -x_18 = lean_array_fget(x_4, x_6); -x_19 = lean_ctor_get(x_18, 0); +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_14 = lean_unsigned_to_nat(1u); +x_15 = lean_nat_sub(x_3, x_14); +lean_dec(x_3); +x_16 = lean_array_fget(x_2, x_4); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +x_19 = lean_ctor_get(x_17, 0); lean_inc(x_19); -x_20 = lean_ctor_get(x_18, 1); +x_20 = lean_ctor_get(x_17, 1); lean_inc(x_20); -lean_dec(x_18); -x_21 = lean_ctor_get(x_19, 0); +lean_dec(x_17); +x_21 = lean_ctor_get(x_19, 1); lean_inc(x_21); -x_22 = lean_ctor_get(x_19, 1); -lean_inc(x_22); lean_dec(x_19); -x_23 = lean_ctor_get(x_21, 1); -lean_inc(x_23); -lean_dec(x_21); -x_24 = lean_ctor_get(x_22, 1); -lean_inc(x_24); -lean_dec(x_22); -lean_inc(x_24); -lean_inc(x_23); -x_25 = l_List_appendTR___rarg(x_23, x_24); -lean_inc(x_20); -lean_inc(x_6); -x_26 = lean_alloc_closure((void*)(l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___boxed), 11, 4); -lean_closure_set(x_26, 0, x_23); -lean_closure_set(x_26, 1, x_24); -lean_closure_set(x_26, 2, x_6); -lean_closure_set(x_26, 3, x_20); -x_27 = 0; -x_28 = lean_box(x_27); -x_29 = lean_alloc_closure((void*)(l_Lean_Meta_lambdaTelescope___at_Lean_PrettyPrinter_Delaborator_returnsPi___spec__1___rarg___boxed), 8, 3); -lean_closure_set(x_29, 0, x_20); -lean_closure_set(x_29, 1, x_26); -lean_closure_set(x_29, 2, x_28); -lean_inc(x_12); -lean_inc(x_11); +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +lean_inc(x_22); +lean_inc(x_21); +x_23 = l_List_appendTR___rarg(x_21, x_22); +lean_inc(x_18); +lean_inc(x_4); +x_24 = lean_alloc_closure((void*)(l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___boxed), 11, 4); +lean_closure_set(x_24, 0, x_21); +lean_closure_set(x_24, 1, x_22); +lean_closure_set(x_24, 2, x_4); +lean_closure_set(x_24, 3, x_18); +x_25 = 0; +x_26 = lean_box(x_25); +x_27 = lean_alloc_closure((void*)(l_Lean_Meta_lambdaTelescope___at_Lean_PrettyPrinter_Delaborator_returnsPi___spec__1___rarg___boxed), 8, 3); +lean_closure_set(x_27, 0, x_18); +lean_closure_set(x_27, 1, x_24); +lean_closure_set(x_27, 2, x_26); lean_inc(x_10); lean_inc(x_9); -x_30 = l_Lean_Meta_withExistingLocalDecls___at_Lean_Meta_Match_Alt_toMessageData___spec__4___rarg(x_25, x_29, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_30) == 0) +lean_inc(x_8); +lean_inc(x_7); +x_28 = l_Lean_Meta_withExistingLocalDecls___at_Lean_Meta_Match_Alt_toMessageData___spec__4___rarg(x_23, x_27, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_28) == 0) { -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_31 = lean_ctor_get(x_30, 0); -lean_inc(x_31); -x_32 = lean_ctor_get(x_30, 1); -lean_inc(x_32); -lean_dec(x_30); -x_33 = lean_nat_add(x_6, x_16); -lean_dec(x_6); -x_34 = lean_array_push(x_8, x_31); -x_5 = x_17; -x_6 = x_33; -x_7 = lean_box(0); -x_8 = x_34; -x_13 = x_32; +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_29 = lean_ctor_get(x_28, 0); +lean_inc(x_29); +x_30 = lean_ctor_get(x_28, 1); +lean_inc(x_30); +lean_dec(x_28); +x_31 = lean_nat_add(x_4, x_14); +lean_dec(x_4); +x_32 = lean_array_push(x_6, x_29); +x_3 = x_15; +x_4 = x_31; +x_5 = lean_box(0); +x_6 = x_32; +x_11 = x_30; goto _start; } else { -uint8_t x_36; -lean_dec(x_17); -lean_dec(x_12); -lean_dec(x_11); +uint8_t x_34; +lean_dec(x_15); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); -x_36 = !lean_is_exclusive(x_30); -if (x_36 == 0) +lean_dec(x_4); +x_34 = !lean_is_exclusive(x_28); +if (x_34 == 0) { -return x_30; +return x_28; } else { -lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_37 = lean_ctor_get(x_30, 0); -x_38 = lean_ctor_get(x_30, 1); -lean_inc(x_38); -lean_inc(x_37); -lean_dec(x_30); -x_39 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_39, 0, x_37); -lean_ctor_set(x_39, 1, x_38); -return x_39; +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_28, 0); +x_36 = lean_ctor_get(x_28, 1); +lean_inc(x_36); +lean_inc(x_35); +lean_dec(x_28); +x_37 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +return x_37; } } } else { -lean_object* x_40; -lean_dec(x_12); -lean_dec(x_11); +lean_object* x_38; lean_dec(x_10); lean_dec(x_9); -lean_dec(x_6); -lean_dec(x_5); -x_40 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_40, 0, x_8); -lean_ctor_set(x_40, 1, x_13); -return x_40; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_4); +lean_dec(x_3); +x_38 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_38, 0, x_6); +lean_ctor_set(x_38, 1, x_11); +return x_38; } } } @@ -22029,7 +21810,7 @@ lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_39 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3(x_1, x_11, x_30, x_35, x_36, x_38, lean_box(0), x_37, x_5, x_6, x_7, x_8, x_31); +x_39 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3(x_35, x_35, x_36, x_38, lean_box(0), x_37, x_5, x_6, x_7, x_8, x_31); lean_dec(x_35); if (lean_obj_tag(x_39) == 0) { @@ -22395,7 +22176,7 @@ lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_116 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3(x_1, x_11, x_107, x_112, x_113, x_115, lean_box(0), x_114, x_5, x_6, x_7, x_8, x_108); +x_116 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3(x_112, x_112, x_113, x_115, lean_box(0), x_114, x_5, x_6, x_7, x_8, x_108); lean_dec(x_112); if (lean_obj_tag(x_116) == 0) { @@ -22793,11 +22574,11 @@ x_6 = l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__ return x_6; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { lean_object* x_15; -x_15 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +x_15 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -22806,11 +22587,11 @@ lean_dec(x_9); return x_15; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { lean_object* x_12; -x_12 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_12 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -22819,16 +22600,14 @@ lean_dec(x_6); return x_12; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_14; -x_14 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_4); -lean_dec(x_3); +lean_object* x_12; +x_12 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_2); lean_dec(x_1); -return x_14; +return x_12; } } LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { @@ -25557,7 +25336,7 @@ lean_dec(x_3); return x_9; } } -static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__1() { +static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -25567,27 +25346,27 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__2() { +static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__1; +x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__1; x_2 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_6____closed__7; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__3() { +static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__2; +x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__2; x_2 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_6____closed__8; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__4() { +static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__4() { _start: { lean_object* x_1; @@ -25595,17 +25374,17 @@ x_1 = lean_mk_string_unchecked("initFn", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__5() { +static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__3; -x_2 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__4; +x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__3; +x_2 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__4; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__6() { +static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__6() { _start: { lean_object* x_1; @@ -25613,47 +25392,47 @@ x_1 = lean_mk_string_unchecked("_@", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__7() { +static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__5; -x_2 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__6; +x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__5; +x_2 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__8() { +static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__7; +x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__7; x_2 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_6____closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__9() { +static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__8; +x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__8; x_2 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_6____closed__7; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__10() { +static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__9; +x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__9; x_2 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_6____closed__8; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__11() { +static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__11() { _start: { lean_object* x_1; @@ -25661,33 +25440,33 @@ x_1 = lean_mk_string_unchecked("_hyg", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__12() { +static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__10; -x_2 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__11; +x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__10; +x_2 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__11; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__13() { +static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__12; -x_2 = lean_unsigned_to_nat(8142u); +x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__12; +x_2 = lean_unsigned_to_nat(8144u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144_(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; x_2 = l_Lean_Meta_IndPredBelow_mkBelow___closed__1; x_3 = 0; -x_4 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__13; +x_4 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__13; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); if (lean_obj_tag(x_5) == 0) { @@ -25956,30 +25735,30 @@ l_Lean_Meta_IndPredBelow_mkBelowMatcher_newMotive___lambda__2___closed__1 = _ini lean_mark_persistent(l_Lean_Meta_IndPredBelow_mkBelowMatcher_newMotive___lambda__2___closed__1); l_Lean_Meta_IndPredBelow_mkBelowMatcher_newMotive___lambda__2___closed__2 = _init_l_Lean_Meta_IndPredBelow_mkBelowMatcher_newMotive___lambda__2___closed__2(); lean_mark_persistent(l_Lean_Meta_IndPredBelow_mkBelowMatcher_newMotive___lambda__2___closed__2); -l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__1 = _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__1(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__1); -l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__2 = _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__2(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__2); -l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__3 = _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__3(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__3); -l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__4 = _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__4(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__4); -l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__1 = _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__1(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__1); -l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__2 = _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__2(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__2); -l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__3 = _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__3(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__3); -l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__4 = _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__4(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__4); -l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__5 = _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__5(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__5); -l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__6 = _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__6(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__6); -l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__7 = _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__7(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__7); -l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__8 = _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__8(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__8); +l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__1 = _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__1(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__1); +l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__2 = _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__2(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__2); +l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__3 = _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__3(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__3); +l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__4 = _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__4(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__4); +l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__1 = _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__1(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__1); +l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__2 = _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__2(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__2); +l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__3 = _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__3(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__3); +l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__4 = _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__4(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__4); +l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__5 = _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__5(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__5); +l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__6 = _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__6(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__6); +l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__7 = _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__7(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__7); +l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__8 = _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__8(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__8); l_Lean_addTrace___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__6___closed__1 = _init_l_Lean_addTrace___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__6___closed__1(); l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__3___lambda__2___closed__1 = _init_l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__3___lambda__2___closed__1(); lean_mark_persistent(l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__3___lambda__2___closed__1); @@ -26029,33 +25808,33 @@ l_Lean_Meta_IndPredBelow_mkBelow___closed__6 = _init_l_Lean_Meta_IndPredBelow_mk lean_mark_persistent(l_Lean_Meta_IndPredBelow_mkBelow___closed__6); l_Lean_Meta_IndPredBelow_mkBelow___closed__7 = _init_l_Lean_Meta_IndPredBelow_mkBelow___closed__7(); lean_mark_persistent(l_Lean_Meta_IndPredBelow_mkBelow___closed__7); -l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__1 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__1(); -lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__1); -l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__2 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__2(); -lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__2); -l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__3 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__3(); -lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__3); -l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__4 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__4(); -lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__4); -l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__5 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__5(); -lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__5); -l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__6 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__6(); -lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__6); -l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__7 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__7(); -lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__7); -l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__8 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__8(); -lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__8); -l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__9 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__9(); -lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__9); -l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__10 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__10(); -lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__10); -l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__11 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__11(); -lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__11); -l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__12 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__12(); -lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__12); -l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__13 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__13(); -lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__13); -if (builtin) {res = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142_(lean_io_mk_world()); +l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__1 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__1(); +lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__1); +l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__2 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__2(); +lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__2); +l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__3 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__3(); +lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__3); +l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__4 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__4(); +lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__4); +l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__5 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__5(); +lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__5); +l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__6 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__6(); +lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__6); +l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__7 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__7(); +lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__7); +l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__8 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__8(); +lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__8); +l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__9 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__9(); +lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__9); +l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__10 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__10(); +lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__10); +l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__11 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__11(); +lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__11); +l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__12 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__12(); +lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__12); +l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__13 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__13(); +lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__13); +if (builtin) {res = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }return lean_io_result_mk_ok(lean_box(0)); diff --git a/stage0/stdlib/Lean/Meta/InferType.c b/stage0/stdlib/Lean/Meta/InferType.c index 3c3d4501331c..7b140e70405c 100644 --- a/stage0/stdlib/Lean/Meta/InferType.c +++ b/stage0/stdlib/Lean/Meta/InferType.c @@ -110,6 +110,7 @@ lean_object* l_instBEqProd___rarg(lean_object*, lean_object*, lean_object*, lean LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_withAppRevAux___at_Lean_Expr_instantiateBetaRevRange_visit___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_forallBoundedTelescope___at_Lean_Meta_arrowDomainsN___spec__6(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_throwFunctionExpected___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_arrowDomainsN___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_InferType_0__Lean_Meta_isArrowProp___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isBVar(lean_object*); uint8_t l_Lean_Expr_hasMVar(lean_object*); @@ -203,14 +204,17 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_InferType_0__Lean_Meta_isArrowTyp static lean_object* l_Lean_Meta_throwFunctionExpected___rarg___closed__1; lean_object* lean_expr_lift_loose_bvars(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_throwFunctionExpected___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_arrowDomainsN___lambda__2___closed__4; lean_object* l_Lean_MVarId_isReadOnlyOrSyntheticOpaque(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Expr_instantiateBetaRevRange___closed__8; +LEAN_EXPORT lean_object* l_Lean_Meta_arrowDomainsN___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_throwIncorrectNumberOfLevels___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Expr_instantiateBetaRevRange_visit___closed__8; lean_object* lean_usize_to_nat(size_t); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_InferType_0__Lean_Meta_inferAppType___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_instInhabitedMetaM___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalContext_mkLocalDecl(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t); +static lean_object* l_Lean_Meta_arrowDomainsN___lambda__2___closed__1; lean_object* l_Lean_MessageData_ofExpr(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_instantiateBetaRevRange___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_InferType_0__Lean_Meta_inferFVarType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -236,6 +240,7 @@ uint8_t lean_nat_dec_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_InferType_0__Lean_Meta_isArrowType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PersistentHashMap_insert___at_Lean_MVarId_assign___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_InferType_0__Lean_Meta_inferAppType___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_arrowDomainsN___lambda__2___closed__2; lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at___private_Lean_Meta_InferType_0__Lean_Meta_inferForallType___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_indentExpr(lean_object*); @@ -257,6 +262,7 @@ LEAN_EXPORT lean_object* lean_infer_type(lean_object*, lean_object*, lean_object lean_object* lean_panic_fn(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_InferType_0__Lean_Meta_inferConstType___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_inferTypeImp_infer___closed__1; +static lean_object* l_Lean_Meta_arrowDomainsN___lambda__2___closed__5; lean_object* lean_nat_sub(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at___private_Lean_Meta_InferType_0__Lean_Meta_checkInferTypeCache___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_getAppFn(lean_object*); @@ -325,9 +331,11 @@ lean_object* l_Lean_PersistentHashMap_getCollisionNodeSize___rarg(lean_object*); lean_object* l_Lean_FVarId_throwUnknown___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_throwUnknownMVar___rarg___closed__1; static lean_object* l_Lean_Meta_throwFunctionExpected___rarg___closed__3; +static lean_object* l_Lean_Meta_arrowDomainsN___lambda__2___closed__3; lean_object* l_Lean_Expr_lam___override(lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l___private_Lean_Meta_InferType_0__Lean_Meta_checkInferTypeCache___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Expr_instantiateBetaRevRange___closed__6; +static lean_object* l_Lean_Meta_arrowDomainsN___lambda__2___closed__6; lean_object* l_Lean_Level_normalize(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_isTypeQuick(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at___private_Lean_Meta_InferType_0__Lean_Meta_checkInferTypeCache___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -337,6 +345,7 @@ lean_object* lean_array_uset(lean_object*, size_t, lean_object*); lean_object* l_Lean_MessageData_ofName(lean_object*); lean_object* lean_array_get(lean_object*, lean_object*, lean_object*); lean_object* lean_expr_instantiate1(lean_object*, lean_object*); +lean_object* l___private_Init_Data_Repr_0__Nat_reprFast(lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Expr_instantiateBetaRevRange_visit___spec__8(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_throwTypeExcepted___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_isProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -22830,14 +22839,14 @@ LEAN_EXPORT lean_object* l_Lean_Meta_arrowDomainsN___lambda__1(lean_object* x_1, _start: { size_t x_9; size_t x_10; lean_object* x_11; -x_9 = lean_array_size(x_2); +x_9 = lean_array_size(x_1); x_10 = 0; lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -lean_inc(x_2); -x_11 = l_Array_mapMUnsafe_map___at_Lean_Meta_arrowDomainsN___spec__1(x_9, x_10, x_2, x_4, x_5, x_6, x_7, x_8); +lean_inc(x_1); +x_11 = l_Array_mapMUnsafe_map___at_Lean_Meta_arrowDomainsN___spec__1(x_9, x_10, x_1, x_4, x_5, x_6, x_7, x_8); if (lean_obj_tag(x_11) == 0) { lean_object* x_12; lean_object* x_13; size_t x_14; lean_object* x_15; lean_object* x_16; @@ -22848,12 +22857,12 @@ lean_inc(x_13); lean_dec(x_11); x_14 = lean_array_size(x_12); x_15 = lean_box(0); -x_16 = l_Array_forInUnsafe_loop___at_Lean_Meta_arrowDomainsN___spec__5(x_1, x_2, x_12, x_14, x_10, x_15, x_4, x_5, x_6, x_7, x_13); +x_16 = l_Array_forInUnsafe_loop___at_Lean_Meta_arrowDomainsN___spec__5(x_2, x_1, x_12, x_14, x_10, x_15, x_4, x_5, x_6, x_7, x_13); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_2); +lean_dec(x_1); if (lean_obj_tag(x_16) == 0) { uint8_t x_17; @@ -22932,15 +22941,133 @@ return x_28; } } } +static lean_object* _init_l_Lean_Meta_arrowDomainsN___lambda__2___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("type ", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_arrowDomainsN___lambda__2___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Meta_arrowDomainsN___lambda__2___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Meta_arrowDomainsN___lambda__2___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" does not have ", 15, 15); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_arrowDomainsN___lambda__2___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Meta_arrowDomainsN___lambda__2___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Meta_arrowDomainsN___lambda__2___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" parameters", 11, 11); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_arrowDomainsN___lambda__2___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Meta_arrowDomainsN___lambda__2___closed__5; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_arrowDomainsN___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; uint8_t x_11; +x_10 = lean_array_get_size(x_3); +x_11 = lean_nat_dec_eq(x_10, x_2); +lean_dec(x_10); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; +lean_dec(x_3); +x_12 = l_Lean_MessageData_ofExpr(x_1); +x_13 = l_Lean_Meta_arrowDomainsN___lambda__2___closed__2; +x_14 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_14, 0, x_13); +lean_ctor_set(x_14, 1, x_12); +x_15 = l_Lean_Meta_arrowDomainsN___lambda__2___closed__4; +x_16 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_16, 0, x_14); +lean_ctor_set(x_16, 1, x_15); +x_17 = l___private_Init_Data_Repr_0__Nat_reprFast(x_2); +x_18 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_18, 0, x_17); +x_19 = l_Lean_MessageData_ofFormat(x_18); +x_20 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_20, 0, x_16); +lean_ctor_set(x_20, 1, x_19); +x_21 = l_Lean_Meta_arrowDomainsN___lambda__2___closed__6; +x_22 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_22, 0, x_20); +lean_ctor_set(x_22, 1, x_21); +x_23 = l_Lean_throwError___at___private_Lean_Meta_InferType_0__Lean_Meta_inferProjType___spec__1(x_22, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_24 = !lean_is_exclusive(x_23); +if (x_24 == 0) +{ +return x_23; +} +else +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_23, 0); +x_26 = lean_ctor_get(x_23, 1); +lean_inc(x_26); +lean_inc(x_25); +lean_dec(x_23); +x_27 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +return x_27; +} +} +else +{ +lean_object* x_28; lean_object* x_29; +lean_dec(x_2); +x_28 = lean_box(0); +x_29 = l_Lean_Meta_arrowDomainsN___lambda__1(x_3, x_1, x_28, x_5, x_6, x_7, x_8, x_9); +return x_29; +} +} +} LEAN_EXPORT lean_object* l_Lean_Meta_arrowDomainsN(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; lean_object* x_9; uint8_t x_10; lean_object* x_11; +lean_inc(x_1); x_8 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_8, 0, x_1); lean_inc(x_2); -x_9 = lean_alloc_closure((void*)(l_Lean_Meta_arrowDomainsN___lambda__1___boxed), 8, 1); +x_9 = lean_alloc_closure((void*)(l_Lean_Meta_arrowDomainsN___lambda__2___boxed), 9, 2); lean_closure_set(x_9, 0, x_2); +lean_closure_set(x_9, 1, x_1); x_10 = 0; x_11 = l_Lean_Meta_forallBoundedTelescope___at_Lean_Meta_arrowDomainsN___spec__6___rarg(x_2, x_8, x_9, x_10, x_3, x_4, x_5, x_6, x_7); return x_11; @@ -23031,6 +23158,15 @@ lean_dec(x_3); return x_9; } } +LEAN_EXPORT lean_object* l_Lean_Meta_arrowDomainsN___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l_Lean_Meta_arrowDomainsN___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_4); +return x_10; +} +} LEAN_EXPORT lean_object* l_Lean_Meta_inferArgumentTypesN(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { @@ -23217,6 +23353,18 @@ l_Array_forInUnsafe_loop___at_Lean_Meta_arrowDomainsN___spec__5___closed__3 = _i lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Meta_arrowDomainsN___spec__5___closed__3); l_Array_forInUnsafe_loop___at_Lean_Meta_arrowDomainsN___spec__5___closed__4 = _init_l_Array_forInUnsafe_loop___at_Lean_Meta_arrowDomainsN___spec__5___closed__4(); lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Meta_arrowDomainsN___spec__5___closed__4); +l_Lean_Meta_arrowDomainsN___lambda__2___closed__1 = _init_l_Lean_Meta_arrowDomainsN___lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Meta_arrowDomainsN___lambda__2___closed__1); +l_Lean_Meta_arrowDomainsN___lambda__2___closed__2 = _init_l_Lean_Meta_arrowDomainsN___lambda__2___closed__2(); +lean_mark_persistent(l_Lean_Meta_arrowDomainsN___lambda__2___closed__2); +l_Lean_Meta_arrowDomainsN___lambda__2___closed__3 = _init_l_Lean_Meta_arrowDomainsN___lambda__2___closed__3(); +lean_mark_persistent(l_Lean_Meta_arrowDomainsN___lambda__2___closed__3); +l_Lean_Meta_arrowDomainsN___lambda__2___closed__4 = _init_l_Lean_Meta_arrowDomainsN___lambda__2___closed__4(); +lean_mark_persistent(l_Lean_Meta_arrowDomainsN___lambda__2___closed__4); +l_Lean_Meta_arrowDomainsN___lambda__2___closed__5 = _init_l_Lean_Meta_arrowDomainsN___lambda__2___closed__5(); +lean_mark_persistent(l_Lean_Meta_arrowDomainsN___lambda__2___closed__5); +l_Lean_Meta_arrowDomainsN___lambda__2___closed__6 = _init_l_Lean_Meta_arrowDomainsN___lambda__2___closed__6(); +lean_mark_persistent(l_Lean_Meta_arrowDomainsN___lambda__2___closed__6); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Lean/Meta/LitValues.c b/stage0/stdlib/Lean/Meta/LitValues.c index 7c4b3e383ab0..af844ecf9a67 100644 --- a/stage0/stdlib/Lean/Meta/LitValues.c +++ b/stage0/stdlib/Lean/Meta/LitValues.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Lean.Meta.LitValues -// Imports: Lean.Meta.Basic +// Imports: Lean.Meta.Basic Init.Control.Option #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -7867,6 +7867,7 @@ return x_7; } } lean_object* initialize_Lean_Meta_Basic(uint8_t builtin, lean_object*); +lean_object* initialize_Init_Control_Option(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Lean_Meta_LitValues(uint8_t builtin, lean_object* w) { lean_object * res; @@ -7875,6 +7876,9 @@ _G_initialized = true; res = initialize_Lean_Meta_Basic(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +res = initialize_Init_Control_Option(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Meta_getOfNatValue_x3f___lambda__1___closed__1 = _init_l_Lean_Meta_getOfNatValue_x3f___lambda__1___closed__1(); lean_mark_persistent(l_Lean_Meta_getOfNatValue_x3f___lambda__1___closed__1); l_Lean_Meta_getOfNatValue_x3f___closed__1 = _init_l_Lean_Meta_getOfNatValue_x3f___closed__1(); diff --git a/stage0/stdlib/Lean/Meta/Match/CaseArraySizes.c b/stage0/stdlib/Lean/Meta/Match/CaseArraySizes.c index d7e869b9374d..56e33ad4b24a 100644 --- a/stage0/stdlib/Lean/Meta/Match/CaseArraySizes.c +++ b/stage0/stdlib/Lean/Meta/Match/CaseArraySizes.c @@ -22,13 +22,14 @@ lean_object* l_Lean_Meta_mkLt(lean_object*, lean_object*, lean_object*, lean_obj lean_object* l_Lean_Meta_mkEqSymm(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isAppOfArity(lean_object*, lean_object*, lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_caseArraySizes___spec__3___boxed(lean_object**); lean_object* l_Lean_MVarId_assertExt(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_caseArraySizes___spec__3___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_FVarSubst_get(lean_object*, lean_object*); lean_object* l_Lean_MVarId_getTag(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_fvarId_x21(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_CaseArraySizes_0__Lean_Meta_introArrayLit_loop___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_caseArraySizes___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_stringToMessageData(lean_object*); static lean_object* l_Lean_Meta_getArrayArgType___closed__6; static lean_object* l___private_Lean_Meta_Match_CaseArraySizes_0__Lean_Meta_introArrayLit_loop___closed__1; @@ -37,6 +38,7 @@ lean_object* l_Lean_Expr_appArg_x21(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_getArrayArgType___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_caseArraySizes___spec__1(size_t, size_t, lean_object*); lean_object* l_Lean_MVarId_assign___at_Lean_Meta_getLevel___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_caseArraySizes___spec__3___boxed(lean_object**); LEAN_EXPORT lean_object* l_Lean_Meta_getArrayArgType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_caseArraySizes___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_caseArraySizes___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -73,13 +75,11 @@ uint8_t lean_nat_dec_eq(lean_object*, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_CaseArraySizes_0__Lean_Meta_introArrayLit___closed__1; lean_object* l_Lean_mkRawNatLit(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_caseArraySizes___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_caseArraySizes___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_CaseArraySizes_0__Lean_Meta_introArrayLit_loop___closed__3; lean_object* l_Lean_indentExpr(lean_object*); lean_object* l_Lean_Meta_mkForallFVars(lean_object*, lean_object*, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_caseArraySizes___spec__3___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_getArrayArgType___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_CaseArraySizes_0__Lean_Meta_mkArrayGetLit___closed__1; @@ -1144,7 +1144,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_caseArraySizes___spec__3___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_caseArraySizes___spec__3___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; @@ -1452,7 +1452,7 @@ return x_72; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_caseArraySizes___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_caseArraySizes___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { _start: { lean_object* x_18; uint8_t x_19; @@ -1622,7 +1622,7 @@ x_58 = l_Lean_Expr_fvar___override(x_26); lean_inc(x_2); lean_inc(x_3); lean_inc(x_56); -x_59 = lean_alloc_closure((void*)(l_Array_mapIdxM_map___at_Lean_Meta_caseArraySizes___spec__3___lambda__1), 12, 7); +x_59 = lean_alloc_closure((void*)(l_Array_mapFinIdxM_map___at_Lean_Meta_caseArraySizes___spec__3___lambda__1), 12, 7); lean_closure_set(x_59, 0, x_58); lean_closure_set(x_59, 1, x_56); lean_closure_set(x_59, 2, x_3); @@ -1929,7 +1929,7 @@ lean_dec(x_38); x_41 = lean_array_get_size(x_39); x_42 = lean_mk_empty_array_with_capacity(x_41); x_43 = lean_unsigned_to_nat(0u); -x_44 = l_Array_mapIdxM_map___at_Lean_Meta_caseArraySizes___spec__3(x_5, x_7, x_8, x_28, x_33, x_36, x_39, x_39, x_41, x_43, lean_box(0), x_42, x_9, x_10, x_11, x_12, x_40); +x_44 = l_Array_mapFinIdxM_map___at_Lean_Meta_caseArraySizes___spec__3(x_5, x_7, x_8, x_28, x_33, x_36, x_39, x_39, x_41, x_43, lean_box(0), x_42, x_9, x_10, x_11, x_12, x_40); lean_dec(x_39); lean_dec(x_5); return x_44; @@ -2163,7 +2163,7 @@ lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_caseArraySizes___spec__3___boxed(lean_object** _args) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_caseArraySizes___spec__3___boxed(lean_object** _args) { lean_object* x_1 = _args[0]; lean_object* x_2 = _args[1]; lean_object* x_3 = _args[2]; @@ -2186,7 +2186,7 @@ lean_object* x_17 = _args[16]; size_t x_18; lean_object* x_19; x_18 = lean_unbox_usize(x_6); lean_dec(x_6); -x_19 = l_Array_mapIdxM_map___at_Lean_Meta_caseArraySizes___spec__3(x_1, x_2, x_3, x_4, x_5, x_18, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +x_19 = l_Array_mapFinIdxM_map___at_Lean_Meta_caseArraySizes___spec__3(x_1, x_2, x_3, x_4, x_5, x_18, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); lean_dec(x_8); lean_dec(x_7); lean_dec(x_1); diff --git a/stage0/stdlib/Lean/Meta/Match/Match.c b/stage0/stdlib/Lean/Meta/Match/Match.c index 151fe1ccc3de..730d254359bd 100644 --- a/stage0/stdlib/Lean/Meta/Match/Match.c +++ b/stage0/stdlib/Lean/Meta/Match/Match.c @@ -33,6 +33,7 @@ static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_throwNo LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_Match_withCleanLCtxFor___spec__18___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Match_mkMatcher___lambda__5___closed__2; static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_hasArrayLitPattern___closed__1; +static lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_Match_getMkMatcherInputInContext___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_constructorApp_x27_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_hasArrayLitPattern___lambda__1(lean_object*); @@ -42,6 +43,7 @@ lean_object* l_Lean_MVarId_contradictionCore(lean_object*, lean_object*, lean_ob LEAN_EXPORT lean_object* l_Lean_Meta_Match_processInaccessibleAsCtor___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkNatLit(lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_throwCasesException___rarg___closed__15; +static lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__2; lean_object* l_instBEqOfDecidableEq___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_expandNatValuePattern___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_process___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -160,9 +162,7 @@ LEAN_EXPORT uint8_t l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_isConst lean_object* lean_mk_array(lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); extern uint8_t l_instInhabitedBool; -static lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__1; static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_hasVarPattern___closed__1; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_withAlts_loop___rarg___closed__5; static lean_object* l_Lean_Meta_Match_mkMatcher___lambda__4___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_Match_mkMatcher(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -225,6 +225,7 @@ static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_expandV lean_object* l_Lean_Meta_getMatcherInfo_x3f___at_Lean_Meta_reduceMatcher_x3f___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Match_processInaccessibleAsCtor(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Match_processInaccessibleAsCtor___lambda__1___closed__2; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Match_withMkMatcherInput___rarg___lambda__1___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_throwCasesException(lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processLeaf___lambda__2___closed__1; @@ -261,6 +262,7 @@ lean_object* l_Lean_RBNode_findCore___at_Lean_Meta_removeUnused___spec__1(lean_o LEAN_EXPORT lean_object* l_Lean_Meta_Match_withMkMatcherInput(lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_throwCasesException___rarg___closed__12; static lean_object* l_List_forIn_loop___at_Lean_Meta_Match_withMkMatcherInput___spec__4___closed__2; +static lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__2; static lean_object* l_Lean_Meta_Match_mkMatcher___lambda__6___closed__5; lean_object* l_Lean_throwError___at_Lean_Meta_setInlineAttribute___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processSkipInaccessible___closed__1; @@ -288,7 +290,6 @@ lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Meta_GeneralizeTelescope_genera static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_traceStep___closed__1; LEAN_EXPORT lean_object* l_List_foldl___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_collectValues___spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_solveSomeLocalFVarIdCnstr_x3f_go___closed__1; -static lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__4; lean_object* l_Lean_Meta_Match_Alt_replaceFVarId(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Match_mkMatcher___lambda__14(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Match_getMkMatcherInputInContext___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -334,6 +335,7 @@ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_Match_withClea LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processLeaf___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_isValueOnlyTransitionCore___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processSkipInaccessible(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_isArrayLitTransition___lambda__1___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_isArrayLitTransition___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_filterTrivialCnstrs___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -358,6 +360,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_ha LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Match_processInaccessibleAsCtor___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_solveSomeLocalFVarIdCnstr_x3f_go___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Match_mkMatcherAuxDefinition___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Match_mkMatcherAuxDefinition(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Meta_Match_withMkMatcherInput___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -372,7 +375,6 @@ LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_ static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_process___closed__4; static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processLeaf_go___closed__1; LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_Match_withCleanLCtxFor___spec__19___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__2; lean_object* l_Lean_Meta_forallBoundedTelescope___at_Lean_Meta_arrowDomainsN___spec__6___rarg(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_checkNextPatternTypes___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -455,6 +457,7 @@ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_Match_withClea LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_solveCnstrs_go___spec__4___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_solveCnstrs_go___closed__3; lean_object* l_Lean_Meta_caseArraySizes(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__1___boxed(lean_object**); LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Meta_Match_mkMatcher___spec__6(lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_expandVarIntoArrayLit_loop___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -503,6 +506,7 @@ static lean_object* l_List_mapM_loop___at___private_Lean_Meta_Match_Match_0__Lea LEAN_EXPORT lean_object* l_Lean_Meta_Match_mkMatcher___lambda__23(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_levelZero; LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_solveSomeLocalFVarIdCnstr_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Meta_Match_mkMatcherAuxDefinition___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processConstructor___closed__2; static lean_object* l_List_forIn_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_checkNextPatternTypes___spec__2___closed__1; @@ -511,6 +515,7 @@ static lean_object* l_List_mapM_loop___at___private_Lean_Meta_Match_Match_0__Lea extern lean_object* l_Lean_instInhabitedExpr; LEAN_EXPORT lean_object* l_Lean_Meta_Match_mkMatcher___lambda__15(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_throwCasesException___rarg___closed__8; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processConstructor___spec__6(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Match_mkMatcher___lambda__18___boxed(lean_object**); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_hasCtorOrInaccessible___lambda__1___boxed(lean_object*); @@ -547,7 +552,6 @@ static lean_object* l_Lean_isTracingEnabledFor___at___private_Lean_Meta_Match_Ma LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___spec__3(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Match_mkMatcherAuxDefinition___lambda__4___closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Meta_Match_withMkMatcherInput___spec__2___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_isBitVecValueTransition___closed__1; LEAN_EXPORT uint8_t l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_inLocalDecls(lean_object*, lean_object*); lean_object* l_instHashableProd___rarg___boxed(lean_object*, lean_object*, lean_object*); @@ -609,6 +613,7 @@ LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_ LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_hasRecursiveType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_solveCnstrs_go___spec__6(lean_object*, lean_object*, lean_object*); static lean_object* l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processSkipInaccessible___spec__3___closed__3; +static lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_isFinValueTransition(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_mapM_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_expandBitVecValuePattern___spec__1___closed__10; static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_solveSomeLocalFVarIdCnstr_x3f___lambda__2___closed__6; @@ -638,9 +643,9 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private static lean_object* l_Lean_Meta_Match_mkMatcher___lambda__2___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_Match_mkMatcher___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_usize_to_nat(size_t); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___boxed(lean_object**); lean_object* l_Lean_Meta_instInhabitedMetaM___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_mapM_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_expandBitVecValuePattern___spec__1___closed__2; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___boxed(lean_object**); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Match_mkMatcher___spec__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkConstWithLevelParams___at_Lean_Meta_mkSimpCongrTheorem___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -653,6 +658,7 @@ LEAN_EXPORT lean_object* l_panic___at___private_Lean_Meta_Match_Match_0__Lean_Me static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_hasAsPattern___closed__1; extern lean_object* l_Lean_inheritedTraceOptions; static lean_object* l_List_mapM_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_expandIntValuePattern___spec__1___closed__5; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofExpr(lean_object*); static lean_object* l_Lean_Meta_Match_getMkMatcherInputInContext___lambda__3___closed__1; lean_object* l_Lean_Option_register___at_Lean_Elab_initFn____x40_Lean_Elab_AutoBound___hyg_6____spec__1(lean_object*, lean_object*, lean_object*, lean_object*); @@ -770,7 +776,6 @@ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_Match_withClea LEAN_EXPORT uint8_t l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_isValueTransition(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Meta_Match_withMkMatcherInput___spec__2(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_isNatValueTransition___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__2; static lean_object* l_List_mapM_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_expandBitVecValuePattern___spec__1___closed__7; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Match_mkMatcher___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_throwCasesException___rarg___closed__2; @@ -839,7 +844,6 @@ lean_object* l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_obj lean_object* l_Array_ofSubarray___rarg(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processVariable(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processLeaf___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_throwCasesException___rarg___closed__3; LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___spec__7(lean_object*, lean_object*, lean_object*); @@ -854,7 +858,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_ex LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_withAlts_loop___rarg___lambda__1___boxed(lean_object**); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_isFirstPatternVar___boxed(lean_object*); size_t lean_usize_sub(size_t, size_t); -static lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__1; lean_object* lean_array_mk(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Match_mkMatcher___lambda__5___boxed(lean_object**); static lean_object* l_Lean_Meta_Match_processInaccessibleAsCtor___lambda__1___closed__3; @@ -863,7 +866,6 @@ extern lean_object* l_Lean_Meta_Match_instInhabitedAlt; static lean_object* l_Lean_Meta_Match_mkMatcherAuxDefinition___lambda__4___closed__1; static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_10875____closed__3; static lean_object* l_Lean_Meta_Match_mkMatcher___lambda__16___closed__1; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__1___boxed(lean_object**); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_process___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static size_t l_Lean_PersistentHashMap_findAux___at_Lean_Meta_Match_mkMatcherAuxDefinition___spec__2___closed__1; LEAN_EXPORT lean_object* l_List_forM___at_Lean_Meta_Match_MkMatcherInput_collectFVars___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -882,7 +884,6 @@ static lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Meta_Match_withMkM LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Meta_Match_mkMatcherAuxDefinition___spec__6(size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_expandVarIntoCtor_x3f___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Match_mkMatcherAuxDefinition___spec__1___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_expandVarIntoCtor_x3f___lambda__2___closed__2; extern lean_object* l_Lean_instInhabitedName; static lean_object* l_List_mapM_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_expandBitVecValuePattern___spec__1___closed__11; @@ -914,7 +915,6 @@ size_t lean_usize_shift_left(size_t, size_t); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_Match_withCleanLCtxFor___spec__21___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_setInlineAttribute(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Match_Match___hyg_14488____closed__12; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_10837____closed__5; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Match_mkMatcher___spec__5(lean_object*, size_t, size_t, lean_object*); @@ -927,7 +927,6 @@ lean_object* l_instDecidableEqNat___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_Match_withCleanLCtxFor___spec__4(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Meta_Match_processInaccessibleAsCtor___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_isTracingEnabledFor___at_Lean_Meta_processPostponed_loop___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__3; LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_Match_withCleanLCtxFor___spec__6(lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* l_List_mapM_loop___at_Lean_Meta_Match_instantiateAltLHSMVars___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processAsPattern___closed__1; @@ -936,6 +935,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_ex LEAN_EXPORT lean_object* l_Lean_Meta_Match_mkMatcher___lambda__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_throwCasesException___rarg___closed__1; static lean_object* l_Lean_Meta_Match_withMkMatcherInput___rarg___lambda__1___closed__2; +static lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_withAlts_loop___rarg___lambda__1(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Meta_Match_mkMatcher___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Match_getMkMatcherInputInContext___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -943,6 +943,7 @@ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_Match_withClea uint8_t l_Lean_isAuxRecursorWithSuffix(lean_object*, lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_10837____closed__3; +static lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__1; static lean_object* l_Lean_Meta_Match_mkMatcher___lambda__6___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_isIntValueTransition(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_int_neg(lean_object*); @@ -971,7 +972,7 @@ lean_object* lean_nat_add(lean_object*, lean_object*); lean_object* l_Lean_PersistentHashMap_getCollisionNodeSize___rarg(lean_object*); LEAN_EXPORT lean_object* l_List_filterTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processConstructor___spec__7___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_isValueTransition___lambda__1(lean_object*); -LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_isConstructorTransition(lean_object*); static lean_object* l_List_mapM_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_expandIntValuePattern___spec__1___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_expandVarIntoCtor_x3f___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -984,7 +985,7 @@ static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_solveSo LEAN_EXPORT lean_object* l_Lean_Meta_Match_mkMatcher___lambda__19___boxed__const__1; LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_withEqs_go___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_checkpointDefEq___at_Lean_Meta_isLevelDefEq___spec__1(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Meta_Match_mkMatcher___spec__15___at_Lean_Meta_Match_mkMatcher___spec__16___at_Lean_Meta_Match_mkMatcher___spec__17(lean_object*, lean_object*); uint8_t l_Lean_Expr_isFVar(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_Match_processInaccessibleAsCtor___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1014,7 +1015,6 @@ lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_instantiateForallAux(lean_ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_Match_withCleanLCtxFor___spec__18(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_isValueOnlyTransitionCore___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_expandVarIntoArrayLit_loop___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processLeaf___lambda__2___closed__2; lean_object* l_Lean_Meta_Match_Alt_toMessageData(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_mapM_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_expandBitVecValuePattern___spec__1___closed__3; @@ -19268,301 +19268,301 @@ x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; } } -LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, uint8_t x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, uint8_t x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, uint8_t x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { -if (lean_obj_tag(x_12) == 0) +if (lean_obj_tag(x_13) == 0) { -lean_object* x_14; -lean_dec(x_9); -x_14 = l_List_reverse___rarg(x_13); -return x_14; +lean_object* x_15; +lean_dec(x_10); +x_15 = l_List_reverse___rarg(x_14); +return x_15; } else { -lean_object* x_15; lean_object* x_16; -x_15 = lean_ctor_get(x_12, 0); -lean_inc(x_15); -x_16 = lean_ctor_get(x_15, 4); +lean_object* x_16; lean_object* x_17; +x_16 = lean_ctor_get(x_13, 0); lean_inc(x_16); -if (lean_obj_tag(x_16) == 0) +x_17 = lean_ctor_get(x_16, 4); +lean_inc(x_17); +if (lean_obj_tag(x_17) == 0) { -uint8_t x_17; -lean_dec(x_15); -x_17 = !lean_is_exclusive(x_12); -if (x_17 == 0) +uint8_t x_18; +lean_dec(x_16); +x_18 = !lean_is_exclusive(x_13); +if (x_18 == 0) { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_18 = lean_ctor_get(x_12, 1); -x_19 = lean_ctor_get(x_12, 0); -lean_dec(x_19); -x_20 = l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7___closed__2; -x_21 = l_panic___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__6(x_20); -lean_ctor_set(x_12, 1, x_13); -lean_ctor_set(x_12, 0, x_21); -{ -lean_object* _tmp_7 = lean_box(0); -lean_object* _tmp_11 = x_18; -lean_object* _tmp_12 = x_12; -x_8 = _tmp_7; -x_12 = _tmp_11; +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_19 = lean_ctor_get(x_13, 1); +x_20 = lean_ctor_get(x_13, 0); +lean_dec(x_20); +x_21 = l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7___closed__2; +x_22 = l_panic___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__6(x_21); +lean_ctor_set(x_13, 1, x_14); +lean_ctor_set(x_13, 0, x_22); +{ +lean_object* _tmp_8 = lean_box(0); +lean_object* _tmp_12 = x_19; +lean_object* _tmp_13 = x_13; +x_9 = _tmp_8; x_13 = _tmp_12; +x_14 = _tmp_13; } goto _start; } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_23 = lean_ctor_get(x_12, 1); -lean_inc(x_23); -lean_dec(x_12); -x_24 = l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7___closed__2; -x_25 = l_panic___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__6(x_24); -x_26 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_26, 1, x_13); -x_8 = lean_box(0); -x_12 = x_23; -x_13 = x_26; +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_24 = lean_ctor_get(x_13, 1); +lean_inc(x_24); +lean_dec(x_13); +x_25 = l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7___closed__2; +x_26 = l_panic___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__6(x_25); +x_27 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_14); +x_9 = lean_box(0); +x_13 = x_24; +x_14 = x_27; goto _start; } } else { -lean_object* x_28; -x_28 = lean_ctor_get(x_16, 0); -lean_inc(x_28); -switch (lean_obj_tag(x_28)) { +lean_object* x_29; +x_29 = lean_ctor_get(x_17, 0); +lean_inc(x_29); +switch (lean_obj_tag(x_29)) { case 1: { -lean_object* x_29; uint8_t x_30; -x_29 = lean_ctor_get(x_12, 1); -lean_inc(x_29); -lean_dec(x_12); -x_30 = !lean_is_exclusive(x_15); -if (x_30 == 0) +lean_object* x_30; uint8_t x_31; +x_30 = lean_ctor_get(x_13, 1); +lean_inc(x_30); +lean_dec(x_13); +x_31 = !lean_is_exclusive(x_16); +if (x_31 == 0) { -lean_object* x_31; uint8_t x_32; -x_31 = lean_ctor_get(x_15, 4); -lean_dec(x_31); -x_32 = !lean_is_exclusive(x_16); -if (x_32 == 0) +lean_object* x_32; uint8_t x_33; +x_32 = lean_ctor_get(x_16, 4); +lean_dec(x_32); +x_33 = !lean_is_exclusive(x_17); +if (x_33 == 0) { -lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_33 = lean_ctor_get(x_16, 1); -x_34 = lean_ctor_get(x_16, 0); -lean_dec(x_34); -x_35 = lean_ctor_get(x_28, 0); -lean_inc(x_35); -lean_dec(x_28); -lean_ctor_set(x_15, 4, x_33); -lean_inc(x_9); -x_36 = l_Lean_Meta_Match_Alt_replaceFVarId(x_35, x_9, x_15); -lean_ctor_set(x_16, 1, x_13); -lean_ctor_set(x_16, 0, x_36); -x_8 = lean_box(0); -x_12 = x_29; -x_13 = x_16; +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_34 = lean_ctor_get(x_17, 1); +x_35 = lean_ctor_get(x_17, 0); +lean_dec(x_35); +x_36 = lean_ctor_get(x_29, 0); +lean_inc(x_36); +lean_dec(x_29); +lean_ctor_set(x_16, 4, x_34); +lean_inc(x_10); +x_37 = l_Lean_Meta_Match_Alt_replaceFVarId(x_36, x_10, x_16); +lean_ctor_set(x_17, 1, x_14); +lean_ctor_set(x_17, 0, x_37); +x_9 = lean_box(0); +x_13 = x_30; +x_14 = x_17; goto _start; } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_38 = lean_ctor_get(x_16, 1); -lean_inc(x_38); -lean_dec(x_16); -x_39 = lean_ctor_get(x_28, 0); +lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_39 = lean_ctor_get(x_17, 1); lean_inc(x_39); -lean_dec(x_28); -lean_ctor_set(x_15, 4, x_38); -lean_inc(x_9); -x_40 = l_Lean_Meta_Match_Alt_replaceFVarId(x_39, x_9, x_15); -x_41 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_41, 0, x_40); -lean_ctor_set(x_41, 1, x_13); -x_8 = lean_box(0); -x_12 = x_29; -x_13 = x_41; +lean_dec(x_17); +x_40 = lean_ctor_get(x_29, 0); +lean_inc(x_40); +lean_dec(x_29); +lean_ctor_set(x_16, 4, x_39); +lean_inc(x_10); +x_41 = l_Lean_Meta_Match_Alt_replaceFVarId(x_40, x_10, x_16); +x_42 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_42, 0, x_41); +lean_ctor_set(x_42, 1, x_14); +x_9 = lean_box(0); +x_13 = x_30; +x_14 = x_42; goto _start; } } else { -lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; -x_43 = lean_ctor_get(x_15, 0); -x_44 = lean_ctor_get(x_15, 1); -x_45 = lean_ctor_get(x_15, 2); -x_46 = lean_ctor_get(x_15, 3); -x_47 = lean_ctor_get(x_15, 5); +lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_44 = lean_ctor_get(x_16, 0); +x_45 = lean_ctor_get(x_16, 1); +x_46 = lean_ctor_get(x_16, 2); +x_47 = lean_ctor_get(x_16, 3); +x_48 = lean_ctor_get(x_16, 5); +lean_inc(x_48); lean_inc(x_47); lean_inc(x_46); lean_inc(x_45); lean_inc(x_44); -lean_inc(x_43); -lean_dec(x_15); -x_48 = lean_ctor_get(x_16, 1); -lean_inc(x_48); -if (lean_is_exclusive(x_16)) { - lean_ctor_release(x_16, 0); - lean_ctor_release(x_16, 1); - x_49 = x_16; +lean_dec(x_16); +x_49 = lean_ctor_get(x_17, 1); +lean_inc(x_49); +if (lean_is_exclusive(x_17)) { + lean_ctor_release(x_17, 0); + lean_ctor_release(x_17, 1); + x_50 = x_17; } else { - lean_dec_ref(x_16); - x_49 = lean_box(0); + lean_dec_ref(x_17); + x_50 = lean_box(0); } -x_50 = lean_ctor_get(x_28, 0); -lean_inc(x_50); -lean_dec(x_28); -x_51 = lean_alloc_ctor(0, 6, 0); -lean_ctor_set(x_51, 0, x_43); -lean_ctor_set(x_51, 1, x_44); -lean_ctor_set(x_51, 2, x_45); -lean_ctor_set(x_51, 3, x_46); -lean_ctor_set(x_51, 4, x_48); -lean_ctor_set(x_51, 5, x_47); -lean_inc(x_9); -x_52 = l_Lean_Meta_Match_Alt_replaceFVarId(x_50, x_9, x_51); -if (lean_is_scalar(x_49)) { - x_53 = lean_alloc_ctor(1, 2, 0); +x_51 = lean_ctor_get(x_29, 0); +lean_inc(x_51); +lean_dec(x_29); +x_52 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_52, 0, x_44); +lean_ctor_set(x_52, 1, x_45); +lean_ctor_set(x_52, 2, x_46); +lean_ctor_set(x_52, 3, x_47); +lean_ctor_set(x_52, 4, x_49); +lean_ctor_set(x_52, 5, x_48); +lean_inc(x_10); +x_53 = l_Lean_Meta_Match_Alt_replaceFVarId(x_51, x_10, x_52); +if (lean_is_scalar(x_50)) { + x_54 = lean_alloc_ctor(1, 2, 0); } else { - x_53 = x_49; + x_54 = x_50; } -lean_ctor_set(x_53, 0, x_52); -lean_ctor_set(x_53, 1, x_13); -x_8 = lean_box(0); -x_12 = x_29; -x_13 = x_53; +lean_ctor_set(x_54, 0, x_53); +lean_ctor_set(x_54, 1, x_14); +x_9 = lean_box(0); +x_13 = x_30; +x_14 = x_54; goto _start; } } case 3: { -lean_object* x_55; uint8_t x_56; -lean_dec(x_28); -x_55 = lean_ctor_get(x_12, 1); -lean_inc(x_55); -lean_dec(x_12); -x_56 = !lean_is_exclusive(x_15); -if (x_56 == 0) +lean_object* x_56; uint8_t x_57; +lean_dec(x_29); +x_56 = lean_ctor_get(x_13, 1); +lean_inc(x_56); +lean_dec(x_13); +x_57 = !lean_is_exclusive(x_16); +if (x_57 == 0) { -lean_object* x_57; uint8_t x_58; -x_57 = lean_ctor_get(x_15, 4); -lean_dec(x_57); -x_58 = !lean_is_exclusive(x_16); -if (x_58 == 0) +lean_object* x_58; uint8_t x_59; +x_58 = lean_ctor_get(x_16, 4); +lean_dec(x_58); +x_59 = !lean_is_exclusive(x_17); +if (x_59 == 0) { -lean_object* x_59; lean_object* x_60; -x_59 = lean_ctor_get(x_16, 1); -x_60 = lean_ctor_get(x_16, 0); -lean_dec(x_60); -lean_ctor_set(x_15, 4, x_59); -lean_ctor_set(x_16, 1, x_13); -lean_ctor_set(x_16, 0, x_15); -x_8 = lean_box(0); -x_12 = x_55; -x_13 = x_16; +lean_object* x_60; lean_object* x_61; +x_60 = lean_ctor_get(x_17, 1); +x_61 = lean_ctor_get(x_17, 0); +lean_dec(x_61); +lean_ctor_set(x_16, 4, x_60); +lean_ctor_set(x_17, 1, x_14); +lean_ctor_set(x_17, 0, x_16); +x_9 = lean_box(0); +x_13 = x_56; +x_14 = x_17; goto _start; } else { -lean_object* x_62; lean_object* x_63; -x_62 = lean_ctor_get(x_16, 1); -lean_inc(x_62); -lean_dec(x_16); -lean_ctor_set(x_15, 4, x_62); -x_63 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_63, 0, x_15); -lean_ctor_set(x_63, 1, x_13); -x_8 = lean_box(0); -x_12 = x_55; -x_13 = x_63; +lean_object* x_63; lean_object* x_64; +x_63 = lean_ctor_get(x_17, 1); +lean_inc(x_63); +lean_dec(x_17); +lean_ctor_set(x_16, 4, x_63); +x_64 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_64, 0, x_16); +lean_ctor_set(x_64, 1, x_14); +x_9 = lean_box(0); +x_13 = x_56; +x_14 = x_64; goto _start; } } else { -lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_65 = lean_ctor_get(x_15, 0); -x_66 = lean_ctor_get(x_15, 1); -x_67 = lean_ctor_get(x_15, 2); -x_68 = lean_ctor_get(x_15, 3); -x_69 = lean_ctor_get(x_15, 5); +lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; +x_66 = lean_ctor_get(x_16, 0); +x_67 = lean_ctor_get(x_16, 1); +x_68 = lean_ctor_get(x_16, 2); +x_69 = lean_ctor_get(x_16, 3); +x_70 = lean_ctor_get(x_16, 5); +lean_inc(x_70); lean_inc(x_69); lean_inc(x_68); lean_inc(x_67); lean_inc(x_66); -lean_inc(x_65); -lean_dec(x_15); -x_70 = lean_ctor_get(x_16, 1); -lean_inc(x_70); -if (lean_is_exclusive(x_16)) { - lean_ctor_release(x_16, 0); - lean_ctor_release(x_16, 1); - x_71 = x_16; +lean_dec(x_16); +x_71 = lean_ctor_get(x_17, 1); +lean_inc(x_71); +if (lean_is_exclusive(x_17)) { + lean_ctor_release(x_17, 0); + lean_ctor_release(x_17, 1); + x_72 = x_17; } else { - lean_dec_ref(x_16); - x_71 = lean_box(0); + lean_dec_ref(x_17); + x_72 = lean_box(0); } -x_72 = lean_alloc_ctor(0, 6, 0); -lean_ctor_set(x_72, 0, x_65); -lean_ctor_set(x_72, 1, x_66); -lean_ctor_set(x_72, 2, x_67); -lean_ctor_set(x_72, 3, x_68); -lean_ctor_set(x_72, 4, x_70); -lean_ctor_set(x_72, 5, x_69); -if (lean_is_scalar(x_71)) { - x_73 = lean_alloc_ctor(1, 2, 0); +x_73 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_73, 0, x_66); +lean_ctor_set(x_73, 1, x_67); +lean_ctor_set(x_73, 2, x_68); +lean_ctor_set(x_73, 3, x_69); +lean_ctor_set(x_73, 4, x_71); +lean_ctor_set(x_73, 5, x_70); +if (lean_is_scalar(x_72)) { + x_74 = lean_alloc_ctor(1, 2, 0); } else { - x_73 = x_71; + x_74 = x_72; } -lean_ctor_set(x_73, 0, x_72); -lean_ctor_set(x_73, 1, x_13); -x_8 = lean_box(0); -x_12 = x_55; -x_13 = x_73; +lean_ctor_set(x_74, 0, x_73); +lean_ctor_set(x_74, 1, x_14); +x_9 = lean_box(0); +x_13 = x_56; +x_14 = x_74; goto _start; } } default: { -uint8_t x_75; -lean_dec(x_28); -lean_dec(x_15); -x_75 = !lean_is_exclusive(x_16); -if (x_75 == 0) +uint8_t x_76; +lean_dec(x_29); +lean_dec(x_16); +x_76 = !lean_is_exclusive(x_17); +if (x_76 == 0) { -lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; -x_76 = lean_ctor_get(x_16, 1); -lean_dec(x_76); -x_77 = lean_ctor_get(x_16, 0); +lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_77 = lean_ctor_get(x_17, 1); lean_dec(x_77); -x_78 = lean_ctor_get(x_12, 1); -lean_inc(x_78); -lean_dec(x_12); -x_79 = l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7___closed__2; -x_80 = l_panic___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__6(x_79); -lean_ctor_set(x_16, 1, x_13); -lean_ctor_set(x_16, 0, x_80); -x_8 = lean_box(0); -x_12 = x_78; -x_13 = x_16; +x_78 = lean_ctor_get(x_17, 0); +lean_dec(x_78); +x_79 = lean_ctor_get(x_13, 1); +lean_inc(x_79); +lean_dec(x_13); +x_80 = l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7___closed__2; +x_81 = l_panic___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__6(x_80); +lean_ctor_set(x_17, 1, x_14); +lean_ctor_set(x_17, 0, x_81); +x_9 = lean_box(0); +x_13 = x_79; +x_14 = x_17; goto _start; } else { -lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; -lean_dec(x_16); -x_82 = lean_ctor_get(x_12, 1); -lean_inc(x_82); -lean_dec(x_12); -x_83 = l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7___closed__2; -x_84 = l_panic___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__6(x_83); -x_85 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_85, 0, x_84); -lean_ctor_set(x_85, 1, x_13); -x_8 = lean_box(0); -x_12 = x_82; -x_13 = x_85; +lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; +lean_dec(x_17); +x_83 = lean_ctor_get(x_13, 1); +lean_inc(x_83); +lean_dec(x_13); +x_84 = l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7___closed__2; +x_85 = l_panic___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__6(x_84); +x_86 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_86, 0, x_85); +lean_ctor_set(x_86, 1, x_14); +x_9 = lean_box(0); +x_13 = x_83; +x_14 = x_86; goto _start; } } @@ -19730,7 +19730,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, uint8_t x_8, lean_object* x_9, uint8_t x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, uint8_t x_8, lean_object* x_9, uint8_t x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19) { _start: { lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; @@ -19748,7 +19748,7 @@ x_25 = l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match x_26 = l_List_filterTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__4(x_1, x_21, x_23); lean_inc(x_4); x_27 = l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__5(x_2, x_5, x_6, x_7, x_8, x_9, lean_box(0), x_4, x_10, x_14, x_26, x_23); -x_28 = l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7(x_2, x_11, x_5, x_6, x_7, x_8, x_9, lean_box(0), x_1, x_10, x_14, x_27, x_23); +x_28 = l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7(x_2, x_11, x_5, x_6, x_7, x_6, x_8, x_9, lean_box(0), x_1, x_10, x_14, x_27, x_23); x_29 = !lean_is_exclusive(x_2); if (x_29 == 0) { @@ -19788,7 +19788,7 @@ return x_38; } } } -static lean_object* _init_l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__1() { +static lean_object* _init_l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__1() { _start: { lean_object* x_1; @@ -19796,16 +19796,16 @@ x_1 = lean_mk_string_unchecked("processValue subst: ", 20, 20); return x_1; } } -static lean_object* _init_l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__2() { +static lean_object* _init_l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__1; +x_1 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__3() { +static lean_object* _init_l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__3() { _start: { lean_object* x_1; @@ -19813,16 +19813,16 @@ x_1 = lean_mk_string_unchecked(", ", 2, 2); return x_1; } } -static lean_object* _init_l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__4() { +static lean_object* _init_l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__3; +x_1 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__3; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, uint8_t x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, uint8_t x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { lean_object* x_17; uint8_t x_18; @@ -19909,7 +19909,7 @@ lean_dec(x_39); x_43 = lean_box(0); x_44 = lean_unbox(x_40); lean_dec(x_40); -x_45 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__1(x_36, x_3, x_8, x_38, x_9, x_2, x_4, x_10, x_11, x_44, x_1, x_6, x_37, x_43, x_12, x_13, x_14, x_15, x_42); +x_45 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__1(x_36, x_3, x_8, x_38, x_9, x_2, x_4, x_10, x_11, x_44, x_1, x_6, x_37, x_43, x_12, x_13, x_14, x_15, x_42); lean_dec(x_4); return x_45; } @@ -19929,11 +19929,11 @@ lean_inc(x_49); x_51 = l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__9(x_49, x_50); x_52 = l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(x_51, x_50); x_53 = l_Lean_MessageData_ofList(x_52); -x_54 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__2; +x_54 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__2; lean_ctor_set_tag(x_39, 7); lean_ctor_set(x_39, 1, x_53); lean_ctor_set(x_39, 0, x_54); -x_55 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__4; +x_55 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__4; x_56 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_56, 0, x_39); lean_ctor_set(x_56, 1, x_55); @@ -19955,7 +19955,7 @@ lean_inc(x_65); lean_dec(x_63); x_66 = lean_unbox(x_40); lean_dec(x_40); -x_67 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__1(x_36, x_3, x_8, x_38, x_9, x_2, x_4, x_10, x_11, x_66, x_1, x_6, x_37, x_64, x_12, x_13, x_14, x_15, x_65); +x_67 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__1(x_36, x_3, x_8, x_38, x_9, x_2, x_4, x_10, x_11, x_66, x_1, x_6, x_37, x_64, x_12, x_13, x_14, x_15, x_65); lean_dec(x_64); lean_dec(x_4); return x_67; @@ -19972,11 +19972,11 @@ lean_inc(x_69); x_71 = l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__9(x_69, x_70); x_72 = l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(x_71, x_70); x_73 = l_Lean_MessageData_ofList(x_72); -x_74 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__2; +x_74 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__2; x_75 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_75, 0, x_74); lean_ctor_set(x_75, 1, x_73); -x_76 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__4; +x_76 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__4; x_77 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_77, 0, x_75); lean_ctor_set(x_77, 1, x_76); @@ -19998,7 +19998,7 @@ lean_inc(x_86); lean_dec(x_84); x_87 = lean_unbox(x_40); lean_dec(x_40); -x_88 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__1(x_36, x_3, x_8, x_38, x_9, x_2, x_4, x_10, x_11, x_87, x_1, x_6, x_37, x_85, x_12, x_13, x_14, x_15, x_86); +x_88 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__1(x_36, x_3, x_8, x_38, x_9, x_2, x_4, x_10, x_11, x_87, x_1, x_6, x_37, x_85, x_12, x_13, x_14, x_15, x_86); lean_dec(x_85); lean_dec(x_4); return x_88; @@ -20007,7 +20007,7 @@ return x_88; } } } -static lean_object* _init_l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__1() { +static lean_object* _init_l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__1() { _start: { lean_object* x_1; @@ -20015,16 +20015,16 @@ x_1 = lean_mk_string_unchecked("processValue subgoal\n", 21, 21); return x_1; } } -static lean_object* _init_l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__2() { +static lean_object* _init_l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__1; +x_1 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { _start: { lean_object* x_18; uint8_t x_19; @@ -20055,7 +20055,7 @@ lean_inc(x_2); lean_inc(x_4); lean_inc(x_3); lean_inc(x_1); -x_29 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2(x_5, x_10, x_1, x_22, x_3, x_4, x_2, x_6, x_7, x_28, x_27, x_13, x_14, x_15, x_16, x_26); +x_29 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2(x_5, x_10, x_1, x_22, x_3, x_4, x_2, x_6, x_7, x_28, x_27, x_13, x_14, x_15, x_16, x_26); x_30 = lean_ctor_get(x_29, 0); lean_inc(x_30); x_31 = lean_ctor_get(x_29, 1); @@ -20085,7 +20085,7 @@ x_38 = lean_ctor_get(x_22, 0); lean_inc(x_38); x_39 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_39, 0, x_38); -x_40 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__2; +x_40 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__2; lean_ctor_set_tag(x_23, 7); lean_ctor_set(x_23, 1, x_39); lean_ctor_set(x_23, 0, x_40); @@ -20106,7 +20106,7 @@ lean_inc(x_2); lean_inc(x_4); lean_inc(x_3); lean_inc(x_1); -x_47 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2(x_5, x_10, x_1, x_22, x_3, x_4, x_2, x_6, x_7, x_46, x_44, x_13, x_14, x_15, x_16, x_45); +x_47 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2(x_5, x_10, x_1, x_22, x_3, x_4, x_2, x_6, x_7, x_46, x_44, x_13, x_14, x_15, x_16, x_45); lean_dec(x_44); x_48 = lean_ctor_get(x_47, 0); lean_inc(x_48); @@ -20133,7 +20133,7 @@ x_54 = lean_ctor_get(x_22, 0); lean_inc(x_54); x_55 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_55, 0, x_54); -x_56 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__2; +x_56 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__2; x_57 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_57, 0, x_56); lean_ctor_set(x_57, 1, x_55); @@ -20154,7 +20154,7 @@ lean_inc(x_2); lean_inc(x_4); lean_inc(x_3); lean_inc(x_1); -x_64 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2(x_5, x_10, x_1, x_22, x_3, x_4, x_2, x_6, x_7, x_63, x_61, x_13, x_14, x_15, x_16, x_62); +x_64 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2(x_5, x_10, x_1, x_22, x_3, x_4, x_2, x_6, x_7, x_63, x_61, x_13, x_14, x_15, x_16, x_62); lean_dec(x_61); x_65 = lean_ctor_get(x_64, 0); lean_inc(x_65); @@ -20250,7 +20250,7 @@ lean_dec(x_19); x_22 = lean_array_get_size(x_20); x_23 = lean_mk_empty_array_with_capacity(x_22); x_24 = lean_unsigned_to_nat(0u); -x_25 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11(x_1, x_2, x_12, x_13, x_14, x_16, x_20, x_20, x_22, x_24, lean_box(0), x_23, x_4, x_5, x_6, x_7, x_21); +x_25 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11(x_1, x_2, x_12, x_13, x_14, x_16, x_20, x_20, x_22, x_24, lean_box(0), x_23, x_4, x_5, x_6, x_7, x_21); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -20397,26 +20397,27 @@ lean_dec(x_1); return x_15; } } -LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { -uint8_t x_14; uint8_t x_15; lean_object* x_16; -x_14 = lean_unbox(x_6); -lean_dec(x_6); -x_15 = lean_unbox(x_10); -lean_dec(x_10); -x_16 = l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7(x_1, x_2, x_3, x_4, x_5, x_14, x_7, x_8, x_9, x_15, x_11, x_12, x_13); -lean_dec(x_11); +uint8_t x_15; uint8_t x_16; lean_object* x_17; +x_15 = lean_unbox(x_7); lean_dec(x_7); +x_16 = lean_unbox(x_11); +lean_dec(x_11); +x_17 = l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7(x_1, x_2, x_3, x_4, x_5, x_6, x_15, x_8, x_9, x_10, x_16, x_12, x_13, x_14); +lean_dec(x_12); +lean_dec(x_8); +lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -return x_16; +return x_17; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__1___boxed(lean_object** _args) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__1___boxed(lean_object** _args) { lean_object* x_1 = _args[0]; lean_object* x_2 = _args[1]; lean_object* x_3 = _args[2]; @@ -20443,7 +20444,7 @@ x_20 = lean_unbox(x_8); lean_dec(x_8); x_21 = lean_unbox(x_10); lean_dec(x_10); -x_22 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_20, x_9, x_21, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19); +x_22 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_20, x_9, x_21, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19); lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -20458,13 +20459,13 @@ lean_dec(x_3); return x_22; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { uint8_t x_17; lean_object* x_18; x_17 = lean_unbox(x_10); lean_dec(x_10); -x_18 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_17, x_11, x_12, x_13, x_14, x_15, x_16); +x_18 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_17, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -20477,7 +20478,7 @@ lean_dec(x_1); return x_18; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___boxed(lean_object** _args) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___boxed(lean_object** _args) { lean_object* x_1 = _args[0]; lean_object* x_2 = _args[1]; lean_object* x_3 = _args[2]; @@ -20498,7 +20499,7 @@ lean_object* x_17 = _args[16]; _start: { lean_object* x_18; -x_18 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +x_18 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); @@ -22413,7 +22414,7 @@ return x_161; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { lean_object* x_17; uint8_t x_18; @@ -22784,7 +22785,7 @@ lean_dec(x_18); x_21 = lean_array_get_size(x_19); x_22 = lean_mk_empty_array_with_capacity(x_21); x_23 = lean_unsigned_to_nat(0u); -x_24 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___spec__9(x_1, x_11, x_12, x_13, x_15, x_19, x_19, x_21, x_23, lean_box(0), x_22, x_3, x_4, x_5, x_6, x_20); +x_24 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___spec__9(x_1, x_11, x_12, x_13, x_15, x_19, x_19, x_21, x_23, lean_box(0), x_22, x_3, x_4, x_5, x_6, x_20); lean_dec(x_19); lean_dec(x_15); lean_dec(x_13); @@ -22917,11 +22918,11 @@ lean_dec(x_1); return x_11; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { lean_object* x_17; -x_17 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___spec__9(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_17 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___spec__9(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -49014,18 +49015,18 @@ l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_proces lean_mark_persistent(l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7___closed__1); l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7___closed__2 = _init_l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7___closed__2(); lean_mark_persistent(l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7___closed__2); -l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__1 = _init_l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__1(); -lean_mark_persistent(l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__1); -l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__2 = _init_l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__2(); -lean_mark_persistent(l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__2); -l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__3 = _init_l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__3(); -lean_mark_persistent(l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__3); -l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__4 = _init_l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__4(); -lean_mark_persistent(l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__4); -l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__1 = _init_l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__1(); -lean_mark_persistent(l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__1); -l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__2 = _init_l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__2(); -lean_mark_persistent(l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__2); +l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__1 = _init_l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__1(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__1); +l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__2 = _init_l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__2(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__2); +l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__3 = _init_l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__3(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__3); +l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__4 = _init_l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__4(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__4); +l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__1 = _init_l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__1(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__1); +l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__2 = _init_l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__2(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__2); l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___lambda__1___closed__1 = _init_l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___lambda__1___closed__1(); lean_mark_persistent(l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___lambda__1___closed__1); l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___closed__1 = _init_l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___closed__1(); diff --git a/stage0/stdlib/Lean/Meta/Offset.c b/stage0/stdlib/Lean/Meta/Offset.c index b941a5596a7a..feb1ebc1aead 100644 --- a/stage0/stdlib/Lean/Meta/Offset.c +++ b/stage0/stdlib/Lean/Meta/Offset.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Lean.Meta.Offset -// Imports: Lean.Data.LBool Lean.Meta.InferType Lean.Meta.NatInstTesters Lean.Util.SafeExponentiation +// Imports: Init.Control.Option Lean.Data.LBool Lean.Meta.InferType Lean.Meta.NatInstTesters Lean.Util.SafeExponentiation #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -10048,6 +10048,7 @@ return x_433; } } } +lean_object* initialize_Init_Control_Option(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Data_LBool(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Meta_InferType(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Meta_NatInstTesters(uint8_t builtin, lean_object*); @@ -10057,6 +10058,9 @@ LEAN_EXPORT lean_object* initialize_Lean_Meta_Offset(uint8_t builtin, lean_objec lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; +res = initialize_Init_Control_Option(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); res = initialize_Lean_Data_LBool(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Lean/Meta/Tactic/AC/Main.c b/stage0/stdlib/Lean/Meta/Tactic/AC/Main.c index 86751a894eda..76a69f296fba 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/AC/Main.c +++ b/stage0/stdlib/Lean/Meta/Tactic/AC/Main.c @@ -17,19 +17,24 @@ static lean_object* l_Std_DHashMap_Internal_AssocList_get_x21___at_Lean_Meta_AC_ lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__9; lean_object* l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_AC_abstractAtoms_go___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_AC_instContextInformationProdPreContextArrayBool___lambda__3___boxed(lean_object*); lean_object* l_Lean_mkNatLit(lean_object*); LEAN_EXPORT lean_object* l_Array_insertionSort_traverse___at_Lean_Meta_AC_toACExpr___spec__7(lean_object*, lean_object*, lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); lean_object* l_Lean_mkAppN(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof___spec__2(size_t, size_t, lean_object*); static lean_object* l_Lean_Meta_AC_buildNormProof_convert___closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_AC_toACExpr(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Std_DHashMap_Internal_AssocList_get_x21___at_Lean_Meta_AC_toACExpr___spec__10___closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_AC_acRflTactic___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Meta_AC_acRflTactic_declRange__1___closed__7; LEAN_EXPORT lean_object* l_Lean_Meta_AC_instEvalInformationPreContextACExpr___lambda__1(lean_object*); +static lean_object* l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__3; static lean_object* l_Lean_Meta_AC_getInstance___closed__6; static lean_object* l_Lean_Meta_AC_buildNormProof_mkContext___closed__6; +LEAN_EXPORT lean_object* l_Lean_Meta_AC_abstractAtoms(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_AC_buildNormProof_mkContext___closed__13; LEAN_EXPORT lean_object* l_Std_HashMap_get_x21___at_Lean_Meta_AC_toACExpr___spec__9___boxed(lean_object*, lean_object*, lean_object*); uint32_t l_UInt32_ofNatTruncate(lean_object*); lean_object* l_Lean_mkApp7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -38,6 +43,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_AC_acNfTargetTactic(lean_object*, lean_obje LEAN_EXPORT lean_object* l_Lean_Meta_AC_acRflTactic(lean_object*); uint8_t l_Lean_Exception_isInterrupt(lean_object*); lean_object* l_Lean_mkAppB(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_AC_buildNormProof___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_ForEachExpr_visit___spec__2(lean_object*, lean_object*); lean_object* l_Lean_Meta_isExprDefEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_getInstance___closed__1; @@ -45,22 +51,27 @@ size_t lean_uint64_to_usize(uint64_t); lean_object* lean_array_fswap(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_preContext___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_AC_rewriteUnnormalized___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t l_Lean_Expr_isAppOfArity(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_expandLocation(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_rewriteUnnormalized___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Elab_Tactic_tacticElabAttribute; static lean_object* l_Lean_Meta_AC_acNfTargetTactic___closed__1; -static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__8; lean_object* lean_array_push(lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_rewriteUnnormalized___closed__12; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof___spec__1(size_t, size_t, lean_object*); +static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__3; +static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__14; lean_object* lean_mk_array(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Meta_AC_acRflTactic__1___closed__8; uint8_t lean_usize_dec_eq(size_t, size_t); extern uint8_t l_instInhabitedBool; LEAN_EXPORT lean_object* l_Lean_Meta_AC_acNfHypMeta___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_rewriteUnnormalized___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__3___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_buildNormProof_convert(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304_(lean_object*); static lean_object* l_Lean_Meta_AC_getInstance___lambda__2___closed__1; +static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__5; +lean_object* l_Lean_Meta_mkExpectedTypeHint(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_bvar___override(lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); lean_object* l_Lean_Meta_Simp_main(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -71,6 +82,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_AC_evalNf0___lambda__4___boxed(lean_object* static lean_object* l_Lean_Meta_AC_rewriteUnnormalized___closed__10; lean_object* l_Lean_Elab_Tactic_getMainGoal(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_AC_toACExpr___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__10; static lean_object* l_Lean_Meta_AC_buildNormProof___closed__1; static lean_object* l_Lean_Meta_AC_buildNormProof_mkContext___closed__11; static lean_object* l___regBuiltin_Lean_Meta_AC_acRflTactic_declRange__1___closed__2; @@ -78,7 +90,6 @@ static lean_object* l_Lean_Meta_AC_preContext___closed__6; static lean_object* l_Lean_Meta_AC_evalNf0___lambda__4___closed__1; static lean_object* l_Lean_Meta_AC_toACExpr___closed__1; lean_object* l_Lean_MVarId_refl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__3; static lean_object* l_Lean_Meta_AC_buildNormProof_mkContext___closed__12; lean_object* l_Lean_addBuiltinDeclarationRanges(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_instContextInformationProdPreContextArrayBool___closed__3; @@ -98,28 +109,31 @@ static lean_object* l___regBuiltin_Lean_Meta_AC_acRflTactic_declRange__1___close lean_object* l_Lean_mkApp4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_getFVarIds(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_acNfHypTactic___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__10; +LEAN_EXPORT lean_object* l_Lean_Data_AC_norm___at_Lean_Meta_AC_buildNormProof___spec__3(lean_object*, lean_object*); lean_object* l_Lean_Meta_getSimpCongrTheorems___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_getInstance___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_evalNf0___closed__3; -static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__2; +static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__11; +lean_object* l_Lean_Expr_appArg_x21(lean_object*); static lean_object* l_Lean_Meta_AC_instContextInformationProdPreContextArrayBool___closed__4; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x21___at_Lean_Meta_AC_toACExpr___spec__10___boxed(lean_object*, lean_object*, lean_object*); extern lean_object* l_instInhabitedNat; -LEAN_EXPORT lean_object* l_Lean_Data_AC_removeNeutrals___at_Lean_Meta_AC_buildNormProof___spec__2___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_preContext___closed__5; -LEAN_EXPORT lean_object* l_Lean_Data_AC_removeNeutrals___at_Lean_Meta_AC_buildNormProof___spec__2(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_AC_buildNormProof___lambda__1___closed__3; +static lean_object* l_Lean_Meta_AC_buildNormProof___lambda__1___closed__4; static lean_object* l___regBuiltin_Lean_Meta_AC_acRflTactic_declRange__1___closed__4; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Meta_AC_toACExpr___spec__2___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_instContextInformationProdPreContextArrayBool___lambda__1(lean_object*, lean_object*); -static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__4; size_t lean_usize_of_nat(lean_object*); +static lean_object* l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__2; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__2; -static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__11; +static lean_object* l_Lean_Meta_AC_buildNormProof___lambda__1___closed__1; lean_object* l_Lean_MVarId_getNondepPropHyps(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_buildNormProof_mkContext(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_panic___rarg(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__1; +LEAN_EXPORT lean_object* l_Lean_Data_AC_norm___at_Lean_Meta_AC_buildNormProof___spec__3___boxed(lean_object*, lean_object*); lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_ForEachExpr_visit___spec__3(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_rewriteUnnormalized___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_evalNf0___closed__1; @@ -132,12 +146,10 @@ LEAN_EXPORT lean_object* l_Lean_Meta_AC_rewriteUnnormalized___lambda__2___boxed( static lean_object* l_Lean_Meta_AC_getInstance___closed__2; static lean_object* l_Lean_Meta_AC_getInstance___closed__7; uint64_t lean_uint64_shift_right(uint64_t, uint64_t); -lean_object* l_Array_unzip___rarg(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_AC_toACExpr___spec__11(lean_object*, size_t, size_t, lean_object*); lean_object* lean_nat_div(lean_object*, lean_object*); lean_object* l_Lean_MVarId_getType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1; -LEAN_EXPORT lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895_(lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__4; static lean_object* l_Lean_Meta_AC_buildNormProof_convert___closed__5; LEAN_EXPORT uint8_t l_Lean_Meta_AC_instContextInformationProdPreContextArrayBool___lambda__3(lean_object*); @@ -145,12 +157,13 @@ static lean_object* l_Lean_Meta_AC_getInstance___lambda__2___closed__2; lean_object* l_Lean_registerTraceClass(lean_object*, uint8_t, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Meta_AC_acRflTactic__1___closed__7; static lean_object* l_Lean_Meta_AC_acNfHypMeta___lambda__1___closed__2; +LEAN_EXPORT lean_object* l_Lean_Data_AC_evalList___at_Lean_Meta_AC_buildNormProof___spec__6(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Meta_AC_acRflTactic_declRange__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Meta_AC_evalNf0___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_buildNormProof_mkContext___closed__8; static lean_object* l_Lean_Meta_AC_buildNormProof___closed__3; static lean_object* l_Lean_Meta_AC_evalNf0___closed__2; -LEAN_EXPORT lean_object* l_Lean_Data_AC_norm___at_Lean_Meta_AC_buildNormProof___spec__1___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__4; lean_object* l_Lean_MVarId_withContext___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_synthPendingImp___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_AC_evalNf0___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Meta_AC_acRflTactic__1___closed__2; @@ -164,13 +177,14 @@ static uint32_t l_Lean_Meta_AC_rewriteUnnormalized___closed__1; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Meta_AC_toACExpr___spec__4(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_evalNf0___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkAppM(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__12; +static lean_object* l_Lean_Meta_AC_buildNormProof___lambda__1___closed__6; static lean_object* l_Lean_Meta_AC_buildNormProof_mkContext___closed__1; +static lean_object* l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__4; static lean_object* l___regBuiltin_Lean_Meta_AC_evalNf0__1___closed__2; lean_object* lean_array_to_list(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_buildNormProof_convertTarget(lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_mkEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_AC_evalNf0___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__3(lean_object*, lean_object*); lean_object* l_Lean_MVarId_withContext___at_Lean_Elab_Tactic_withMainContext___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_evalNf0___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -179,19 +193,21 @@ static lean_object* l_Lean_Meta_AC_rewriteUnnormalized___closed__4; static lean_object* l_Lean_Meta_AC_acNfHypMeta___lambda__1___closed__4; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Meta_AC_toACExpr___spec__6(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_buildNormProof___closed__2; -static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__16; static lean_object* l_Lean_Meta_AC_buildNormProof_convert___closed__2; static lean_object* l_Lean_Meta_AC_acNfHypMeta___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_AC_instContextInformationProdPreContextArrayBool___lambda__2___boxed(lean_object*); static lean_object* l_Lean_Meta_AC_instEvalInformationPreContextACExpr___closed__4; extern lean_object* l_Lean_instInhabitedExpr; +static lean_object* l_Lean_Meta_AC_abstractAtoms_go___closed__2; uint64_t l_Lean_Expr_hash(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__5(lean_object*, lean_object*); lean_object* l_Lean_FVarId_getType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Data_AC_norm___at_Lean_Meta_AC_buildNormProof___spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_panic___at_Lean_Meta_AC_buildNormProof___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Meta_AC_toACExpr___spec__1(lean_object*, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_AC_toACExpr___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_acNfHypMeta___lambda__1___closed__3; +LEAN_EXPORT lean_object* l_Lean_Meta_AC_abstractAtoms_go___lambda__1___boxed(lean_object**); lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__7; lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -201,26 +217,33 @@ uint8_t l_Lean_Syntax_matchesNull(lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_rewriteUnnormalized___closed__9; LEAN_EXPORT lean_object* l_Lean_Meta_AC_acNfHypTactic(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_instEvalInformationPreContextACExpr___lambda__3(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__9; static lean_object* l___regBuiltin_Lean_Meta_AC_acRflTactic__1___closed__3; static lean_object* l___regBuiltin_Lean_Meta_AC_evalNf0__1___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_AC_acRflTactic__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_getInstance___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_AC_toACExpr___spec__12(lean_object*, size_t, size_t, lean_object*); static lean_object* l___regBuiltin_Lean_Meta_AC_evalNf0__1___closed__3; -static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__13; LEAN_EXPORT lean_object* l_Lean_Meta_AC_rewriteUnnormalized___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_rewriteUnnormalized___closed__3; static lean_object* l___regBuiltin_Lean_Meta_AC_acRflTactic_declRange__1___closed__1; +lean_object* l_Lean_Meta_instInhabitedMetaM___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_rewriteUnnormalizedRefl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__15; +static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__8; +lean_object* l_Array_append___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Meta_AC_toACExpr___spec__5(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_buildNormProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_AC_buildNormProof___lambda__1___closed__5; +LEAN_EXPORT lean_object* l_Lean_Meta_AC_buildNormProof___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Data_AC_evalList___at_Lean_Meta_AC_buildNormProof___spec__6___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_toACExpr___closed__4; static lean_object* l_Lean_Meta_AC_preContext___closed__7; uint8_t lean_expr_lt(lean_object*, lean_object*); -static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__7; +LEAN_EXPORT lean_object* l_Lean_Meta_AC_abstractAtoms_go(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__15; LEAN_EXPORT lean_object* l_Lean_Meta_AC_post(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_instEvalInformationPreContextACExpr; +static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__1; lean_object* l_Lean_Data_AC_mergeIdem(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_acRflTactic___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -234,28 +257,32 @@ LEAN_EXPORT lean_object* l_Lean_Meta_AC_buildNormProof_convertTarget___boxed(lea static lean_object* l_Lean_Meta_AC_toACExpr___closed__3; uint8_t lean_nat_dec_eq(lean_object*, lean_object*); lean_object* l_Lean_mkApp3(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__7; LEAN_EXPORT lean_object* l_Lean_Meta_AC_preContext___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_applySimpResultToLocalDecl(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_toACExpr___closed__2; +static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__2; lean_object* l_Lean_instantiateMVars___at___private_Lean_Meta_Basic_0__Lean_Meta_isClassApp_x3f___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkListLit(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Data_AC_removeNeutrals___at_Lean_Meta_AC_buildNormProof___spec__4(lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_instEvalInformationPreContextACExpr___closed__3; -static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__6; LEAN_EXPORT lean_object* l_Lean_Meta_AC_toACExpr_toPreExpr___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_instContextInformationProdPreContextArrayBool___closed__2; lean_object* l_Lean_Meta_mkEqRefl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_AC_abstractAtoms_go___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_indentExpr(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_rewriteUnnormalized___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_panic___at_Lean_Meta_AC_buildNormProof___spec__7___closed__1; +static lean_object* l_Lean_Meta_AC_buildNormProof___lambda__1___closed__2; lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Data_AC_evalList___at_Lean_Meta_AC_buildNormProof___spec__4___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_preContext___closed__3; static lean_object* l_Lean_Meta_AC_buildNormProof_convert___closed__1; static lean_object* l_Lean_Meta_AC_buildNormProof_mkContext___closed__3; uint64_t lean_uint64_xor(uint64_t, uint64_t); uint8_t l_Lean_Syntax_isNone(lean_object*); -static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__9; +lean_object* lean_panic_fn(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_preContext___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_buildNormProof_mkContext___closed__10; static lean_object* l_Lean_Meta_AC_getInstance___closed__3; @@ -263,25 +290,32 @@ lean_object* lean_nat_sub(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Meta_AC_toACExpr___spec__2(lean_object*, lean_object*); lean_object* lean_nat_mul(lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_instEvalInformationPreContextACExpr___lambda__1___closed__1; +static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__16; LEAN_EXPORT lean_object* l_Lean_Meta_AC_getInstance___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__6; lean_object* l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_rewriteUnnormalized___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_instEvalInformationPreContextACExpr___closed__2; LEAN_EXPORT lean_object* l_Array_insertionSort_swapLoop___at_Lean_Meta_AC_toACExpr___spec__8(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_toACExpr_toPreExpr(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__5___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__12; +LEAN_EXPORT lean_object* l_Lean_Meta_AC_abstractAtoms_go___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__6; size_t lean_usize_sub(size_t, size_t); lean_object* lean_array_mk(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_acRflTactic___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_toACExpr_toACExpr(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__13; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x21___at_Lean_Meta_AC_toACExpr___spec__10(lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_SynthInstance_removeUnusedArguments_x3f___spec__2___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_rewriteUnnormalized___closed__11; LEAN_EXPORT lean_object* l_Lean_Meta_AC_instContextInformationProdPreContextArrayBool; static lean_object* l_Lean_Meta_AC_instContextInformationProdPreContextArrayBool___closed__1; LEAN_EXPORT uint8_t l_Lean_Meta_AC_instContextInformationProdPreContextArrayBool___lambda__2(lean_object*); size_t lean_usize_add(size_t, size_t); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Meta_AC_toACExpr___spec__3(lean_object*); -static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__11; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof___spec__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_instInhabitedPreContext___closed__2; static lean_object* l_Lean_Meta_AC_rewriteUnnormalized___closed__8; LEAN_EXPORT lean_object* l_Lean_Meta_AC_instInhabitedPreContext; @@ -296,25 +330,24 @@ LEAN_EXPORT lean_object* l_Lean_Meta_AC_instEvalInformationPreContextACExpr___la static lean_object* l___regBuiltin_Lean_Meta_AC_acRflTactic__1___closed__6; static lean_object* l___regBuiltin_Lean_Meta_AC_acRflTactic_declRange__1___closed__5; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__8; -static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__12; LEAN_EXPORT lean_object* l_Lean_Meta_AC_acRflTactic___boxed(lean_object*); static lean_object* l_Lean_Meta_AC_preContext___closed__8; lean_object* l_Lean_isTracingEnabledFor___at_Lean_Meta_processPostponed_loop___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_post___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_AC_evalNf0__1(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Data_AC_removeNeutrals___at_Lean_Meta_AC_buildNormProof___spec__4___boxed(lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_preContext(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_buildNormProof_mkContext___closed__9; -static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__5; LEAN_EXPORT lean_object* l_Lean_Meta_AC_getInstance___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Meta_AC_acNfTargetTactic___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Data_AC_evalList___at_Lean_Meta_AC_buildNormProof___spec__4(lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_buildNormProof___closed__5; LEAN_EXPORT lean_object* l_Lean_Meta_AC_instEvalInformationPreContextACExpr___lambda__2___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_buildNormProof___closed__6; +lean_object* l_Lean_Meta_mkLambdaFVars(lean_object*, lean_object*, uint8_t, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Std_DHashMap_Internal_AssocList_get_x21___at_Lean_Meta_AC_toACExpr___spec__10___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_AC_toACExpr_toPreExpr___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); @@ -324,6 +357,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_AC_evalNf0___lambda__1(lean_object*, lean_o lean_object* l_Lean_Data_AC_sort(lean_object*); static lean_object* l_Std_DHashMap_Internal_AssocList_get_x21___at_Lean_Meta_AC_toACExpr___spec__10___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_AC_instEvalInformationPreContextACExpr___lambda__3___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof___spec__2___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_buildNormProof_mkContext___closed__7; static lean_object* l_Lean_Meta_AC_getInstance___closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_AC_getInstance(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -333,13 +367,11 @@ lean_object* lean_array_uset(lean_object*, size_t, lean_object*); lean_object* l_Lean_Elab_Tactic_replaceMainGoal(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_buildNormProof_convert___closed__3; static lean_object* l_Lean_Meta_AC_instInhabitedPreContext___closed__1; -static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__14; static lean_object* l_Lean_Meta_AC_buildNormProof_convert___closed__7; static lean_object* l_Lean_Meta_AC_preContext___closed__4; size_t lean_usize_land(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Meta_AC_post___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_getInstance___closed__5; -static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_AC_instContextInformationProdPreContextArrayBool___lambda__1___boxed(lean_object*, lean_object*); static lean_object* _init_l_Lean_Meta_AC_instInhabitedPreContext___closed__1() { _start: @@ -3496,7 +3528,44 @@ lean_dec(x_1); return x_7; } } -static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1() { +LEAN_EXPORT lean_object* l_Lean_Meta_AC_abstractAtoms_go___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19) { +_start: +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_20 = lean_unsigned_to_nat(1u); +x_21 = lean_nat_add(x_1, x_20); +lean_inc(x_14); +x_22 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_22, 0, x_14); +lean_inc(x_2); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_2); +lean_ctor_set(x_23, 1, x_22); +x_24 = lean_array_push(x_3, x_23); +lean_inc(x_4); +x_25 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_25, 0, x_14); +lean_ctor_set(x_25, 1, x_4); +x_26 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_26, 0, x_2); +lean_ctor_set(x_26, 1, x_25); +x_27 = lean_array_mk(x_26); +x_28 = l_Array_append___rarg(x_5, x_27); +lean_dec(x_27); +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_6); +lean_ctor_set(x_29, 1, x_4); +x_30 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_30, 0, x_7); +lean_ctor_set(x_30, 1, x_29); +x_31 = lean_array_mk(x_30); +x_32 = l_Array_append___rarg(x_8, x_31); +lean_dec(x_31); +x_33 = l_Lean_Meta_AC_abstractAtoms_go(x_9, x_10, x_11, x_12, x_13, x_21, x_24, x_28, x_32, x_15, x_16, x_17, x_18, x_19); +return x_33; +} +} +static lean_object* _init_l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__1() { _start: { lean_object* x_1; @@ -3504,481 +3573,425 @@ x_1 = lean_mk_string_unchecked("LawfulIdentity", 14, 14); return x_1; } } -static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__2() { +static lean_object* _init_l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Meta_AC_preContext___closed__1; -x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1; +x_2 = l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__1; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__3() { +static lean_object* _init_l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__3() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("Lean", 4, 4); +x_1 = lean_mk_string_unchecked("inst", 4, 4); return x_1; } } -static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__4() { +static lean_object* _init_l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__4() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Data", 4, 4); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__3; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__5() { +LEAN_EXPORT lean_object* l_Lean_Meta_AC_abstractAtoms_go___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Variable", 8, 8); -return x_1; -} -} -static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__6() { -_start: +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_16 = lean_ctor_get(x_1, 1); +lean_inc(x_16); +x_17 = lean_array_fget(x_2, x_3); +x_18 = lean_box(0); +lean_inc(x_17); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set(x_19, 1, x_18); +lean_inc(x_16); +x_20 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_20, 0, x_16); +lean_ctor_set(x_20, 1, x_19); +x_21 = lean_array_mk(x_20); +x_22 = l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__2; +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +x_23 = l_Lean_Meta_AC_getInstance(x_22, x_21, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_23) == 0) { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("mk", 2, 2); -return x_1; -} +lean_object* x_24; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +if (lean_obj_tag(x_24) == 0) +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +lean_dec(x_16); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +x_26 = lean_unsigned_to_nat(1u); +x_27 = lean_nat_add(x_3, x_26); +lean_dec(x_3); +x_28 = lean_box(0); +lean_inc(x_10); +x_29 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_29, 0, x_10); +lean_ctor_set(x_29, 1, x_28); +x_30 = lean_array_push(x_4, x_29); +x_31 = lean_array_push(x_5, x_10); +x_32 = lean_array_push(x_6, x_17); +x_33 = l_Lean_Meta_AC_abstractAtoms_go(x_1, x_2, x_7, x_8, x_9, x_27, x_30, x_31, x_32, x_11, x_12, x_13, x_14, x_25); +return x_33; } -static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__7() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__3; -x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__4; -x_3 = l_Lean_Meta_AC_getInstance___closed__2; -x_4 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__5; -x_5 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__6; -x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); -return x_6; +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; uint8_t x_42; lean_object* x_43; +x_34 = lean_ctor_get(x_23, 1); +lean_inc(x_34); +lean_dec(x_23); +x_35 = lean_ctor_get(x_24, 0); +lean_inc(x_35); +lean_dec(x_24); +lean_inc(x_9); +x_36 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_36, 0, x_9); +lean_ctor_set(x_36, 1, x_18); +x_37 = l_Lean_Expr_const___override(x_22, x_36); +lean_inc(x_10); +lean_inc(x_8); +x_38 = l_Lean_mkApp3(x_37, x_8, x_16, x_10); +x_39 = lean_alloc_closure((void*)(l_Lean_Meta_AC_abstractAtoms_go___lambda__1___boxed), 19, 13); +lean_closure_set(x_39, 0, x_3); +lean_closure_set(x_39, 1, x_10); +lean_closure_set(x_39, 2, x_4); +lean_closure_set(x_39, 3, x_18); +lean_closure_set(x_39, 4, x_5); +lean_closure_set(x_39, 5, x_35); +lean_closure_set(x_39, 6, x_17); +lean_closure_set(x_39, 7, x_6); +lean_closure_set(x_39, 8, x_1); +lean_closure_set(x_39, 9, x_2); +lean_closure_set(x_39, 10, x_7); +lean_closure_set(x_39, 11, x_8); +lean_closure_set(x_39, 12, x_9); +x_40 = l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__4; +x_41 = 0; +x_42 = 0; +x_43 = l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_SynthInstance_removeUnusedArguments_x3f___spec__2___rarg(x_40, x_41, x_38, x_39, x_42, x_11, x_12, x_13, x_14, x_34); +return x_43; } } -static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__8() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Option", 6, 6); -return x_1; -} +uint8_t x_44; +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_44 = !lean_is_exclusive(x_23); +if (x_44 == 0) +{ +return x_23; } -static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__9() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("none", 4, 4); -return x_1; +lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_45 = lean_ctor_get(x_23, 0); +x_46 = lean_ctor_get(x_23, 1); +lean_inc(x_46); +lean_inc(x_45); +lean_dec(x_23); +x_47 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_47, 0, x_45); +lean_ctor_set(x_47, 1, x_46); +return x_47; } } -static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__10() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__8; -x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__9; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; } } -static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__11() { +static lean_object* _init_l_Lean_Meta_AC_abstractAtoms_go___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("some", 4, 4); +x_1 = lean_mk_string_unchecked("x", 1, 1); return x_1; } } -static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__12() { +static lean_object* _init_l_Lean_Meta_AC_abstractAtoms_go___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__8; -x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__11; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); +x_1 = lean_box(0); +x_2 = l_Lean_Meta_AC_abstractAtoms_go___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, size_t x_8, size_t x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +LEAN_EXPORT lean_object* l_Lean_Meta_AC_abstractAtoms_go(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { -uint8_t x_16; -x_16 = lean_usize_dec_lt(x_9, x_8); +lean_object* x_15; uint8_t x_16; +x_15 = lean_array_get_size(x_2); +x_16 = lean_nat_dec_lt(x_6, x_15); +lean_dec(x_15); if (x_16 == 0) { lean_object* x_17; -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_10); -lean_ctor_set(x_17, 1, x_15); -return x_17; -} -else -{ -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_18 = lean_array_uget(x_10, x_9); -x_19 = lean_unsigned_to_nat(0u); -x_20 = lean_array_uset(x_10, x_9, x_19); -x_21 = lean_ctor_get(x_1, 1); -lean_inc(x_21); -x_22 = lean_box(0); -lean_inc(x_18); -x_23 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_23, 0, x_18); -lean_ctor_set(x_23, 1, x_22); -lean_inc(x_21); -x_24 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_24, 0, x_21); -lean_ctor_set(x_24, 1, x_23); -x_25 = lean_array_mk(x_24); -x_26 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__2; -lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); -x_27 = l_Lean_Meta_AC_getInstance(x_26, x_25, x_11, x_12, x_13, x_14, x_15); -if (lean_obj_tag(x_27) == 0) +lean_inc(x_10); +x_17 = lean_apply_6(x_3, x_7, x_10, x_11, x_12, x_13, x_14); +if (lean_obj_tag(x_17) == 0) { -lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_28 = lean_ctor_get(x_27, 0); -lean_inc(x_28); -x_29 = lean_ctor_get(x_27, 1); -lean_inc(x_29); -lean_dec(x_27); -lean_inc(x_4); -lean_inc(x_3); -x_30 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_30, 0, x_3); -lean_ctor_set(x_30, 1, x_4); -lean_inc(x_30); -x_31 = l_Lean_Expr_const___override(x_26, x_30); +lean_object* x_18; lean_object* x_19; uint8_t x_20; uint8_t x_21; uint8_t x_22; lean_object* x_23; +x_18 = lean_ctor_get(x_17, 0); lean_inc(x_18); -lean_inc(x_21); -lean_inc(x_2); -x_32 = l_Lean_mkApp3(x_31, x_2, x_21, x_18); -x_33 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__7; -x_34 = l_Lean_Expr_const___override(x_33, x_30); -if (lean_obj_tag(x_28) == 0) +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); +lean_dec(x_17); +x_20 = 0; +x_21 = 1; +x_22 = 1; +x_23 = l_Lean_Meta_mkLambdaFVars(x_8, x_18, x_20, x_21, x_20, x_22, x_10, x_11, x_12, x_13, x_19); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +if (lean_obj_tag(x_23) == 0) { -lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; lean_object* x_41; lean_object* x_42; size_t x_43; size_t x_44; lean_object* x_45; -x_35 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__10; -lean_inc(x_5); -x_36 = l_Lean_Expr_const___override(x_35, x_5); -lean_inc(x_6); -x_37 = l_Lean_Expr_app___override(x_6, x_32); -x_38 = l_Lean_Expr_app___override(x_36, x_37); -lean_inc(x_2); -x_39 = l_Lean_mkApp4(x_34, x_2, x_21, x_18, x_38); -x_40 = 0; -x_41 = lean_box(x_40); -x_42 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_42, 0, x_41); -lean_ctor_set(x_42, 1, x_39); -x_43 = 1; -x_44 = lean_usize_add(x_9, x_43); -x_45 = lean_array_uset(x_20, x_9, x_42); -x_9 = x_44; -x_10 = x_45; -x_15 = x_29; -goto _start; +uint8_t x_24; +x_24 = !lean_is_exclusive(x_23); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; +x_25 = lean_ctor_get(x_23, 0); +x_26 = l_Lean_mkAppN(x_25, x_9); +lean_dec(x_9); +lean_ctor_set(x_23, 0, x_26); +return x_23; } else { -lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; uint8_t x_54; lean_object* x_55; lean_object* x_56; size_t x_57; size_t x_58; lean_object* x_59; -x_47 = lean_ctor_get(x_28, 0); -lean_inc(x_47); -lean_dec(x_28); -x_48 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__12; -lean_inc(x_5); -x_49 = l_Lean_Expr_const___override(x_48, x_5); -lean_inc(x_32); -lean_inc(x_6); -x_50 = l_Lean_Expr_app___override(x_6, x_32); -lean_inc(x_7); -x_51 = l_Lean_mkAppB(x_7, x_32, x_47); -x_52 = l_Lean_mkAppB(x_49, x_50, x_51); -lean_inc(x_2); -x_53 = l_Lean_mkApp4(x_34, x_2, x_21, x_18, x_52); -x_54 = 1; -x_55 = lean_box(x_54); -x_56 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_56, 0, x_55); -lean_ctor_set(x_56, 1, x_53); -x_57 = 1; -x_58 = lean_usize_add(x_9, x_57); -x_59 = lean_array_uset(x_20, x_9, x_56); -x_9 = x_58; -x_10 = x_59; -x_15 = x_29; -goto _start; +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_27 = lean_ctor_get(x_23, 0); +x_28 = lean_ctor_get(x_23, 1); +lean_inc(x_28); +lean_inc(x_27); +lean_dec(x_23); +x_29 = l_Lean_mkAppN(x_27, x_9); +lean_dec(x_9); +x_30 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_30, 0, x_29); +lean_ctor_set(x_30, 1, x_28); +return x_30; } } else { -uint8_t x_61; -lean_dec(x_21); -lean_dec(x_20); -lean_dec(x_18); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_61 = !lean_is_exclusive(x_27); -if (x_61 == 0) +uint8_t x_31; +lean_dec(x_9); +x_31 = !lean_is_exclusive(x_23); +if (x_31 == 0) { -return x_27; +return x_23; } else { -lean_object* x_62; lean_object* x_63; lean_object* x_64; -x_62 = lean_ctor_get(x_27, 0); -x_63 = lean_ctor_get(x_27, 1); -lean_inc(x_63); -lean_inc(x_62); -lean_dec(x_27); -x_64 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_64, 0, x_62); -lean_ctor_set(x_64, 1, x_63); -return x_64; -} -} +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_23, 0); +x_33 = lean_ctor_get(x_23, 1); +lean_inc(x_33); +lean_inc(x_32); +lean_dec(x_23); +x_34 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_34, 0, x_32); +lean_ctor_set(x_34, 1, x_33); +return x_34; } } } -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("PLift", 5, 5); -return x_1; -} -} -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = lean_box(0); -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; -} -} -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__2; -x_2 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__3; -x_3 = l_Lean_Expr_const___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__5() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("up", 2, 2); -return x_1; -} -} -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__6() { -_start: +uint8_t x_35; +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +x_35 = !lean_is_exclusive(x_17); +if (x_35 == 0) { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__1; -x_2 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__5; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; -} +return x_17; } -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__7() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__6; -x_2 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__3; -x_3 = l_Lean_Expr_const___override(x_1, x_2); -return x_3; -} +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_17, 0); +x_37 = lean_ctor_get(x_17, 1); +lean_inc(x_37); +lean_inc(x_36); +lean_dec(x_17); +x_38 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_38, 0, x_36); +lean_ctor_set(x_38, 1, x_37); +return x_38; } -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__8() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__3; -x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__4; -x_3 = l_Lean_Meta_AC_getInstance___closed__2; -x_4 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__5; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; } } -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__9() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Context", 7, 7); -return x_1; -} +lean_object* x_39; lean_object* x_40; uint8_t x_41; uint8_t x_42; lean_object* x_43; +lean_inc(x_4); +x_39 = lean_alloc_closure((void*)(l_Lean_Meta_AC_abstractAtoms_go___lambda__2), 15, 9); +lean_closure_set(x_39, 0, x_1); +lean_closure_set(x_39, 1, x_2); +lean_closure_set(x_39, 2, x_6); +lean_closure_set(x_39, 3, x_7); +lean_closure_set(x_39, 4, x_8); +lean_closure_set(x_39, 5, x_9); +lean_closure_set(x_39, 6, x_3); +lean_closure_set(x_39, 7, x_4); +lean_closure_set(x_39, 8, x_5); +x_40 = l_Lean_Meta_AC_abstractAtoms_go___closed__2; +x_41 = 0; +x_42 = 0; +x_43 = l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_SynthInstance_removeUnusedArguments_x3f___spec__2___rarg(x_40, x_41, x_4, x_39, x_42, x_10, x_11, x_12, x_13, x_14); +return x_43; } -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__10() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__3; -x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__4; -x_3 = l_Lean_Meta_AC_getInstance___closed__2; -x_4 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__9; -x_5 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__6; -x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); -return x_6; } } -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__11() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__10; -x_2 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__3; -x_3 = l_Lean_Expr_const___override(x_1, x_2); -return x_3; +LEAN_EXPORT lean_object* l_Lean_Meta_AC_abstractAtoms_go___lambda__1___boxed(lean_object** _args) { +lean_object* x_1 = _args[0]; +lean_object* x_2 = _args[1]; +lean_object* x_3 = _args[2]; +lean_object* x_4 = _args[3]; +lean_object* x_5 = _args[4]; +lean_object* x_6 = _args[5]; +lean_object* x_7 = _args[6]; +lean_object* x_8 = _args[7]; +lean_object* x_9 = _args[8]; +lean_object* x_10 = _args[9]; +lean_object* x_11 = _args[10]; +lean_object* x_12 = _args[11]; +lean_object* x_13 = _args[12]; +lean_object* x_14 = _args[13]; +lean_object* x_15 = _args[14]; +lean_object* x_16 = _args[15]; +lean_object* x_17 = _args[16]; +lean_object* x_18 = _args[17]; +lean_object* x_19 = _args[18]; +_start: +{ +lean_object* x_20; +x_20 = l_Lean_Meta_AC_abstractAtoms_go___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19); +lean_dec(x_1); +return x_20; } } -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__12() { +LEAN_EXPORT lean_object* l_Lean_Meta_AC_abstractAtoms(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__12; -x_2 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__3; -x_3 = l_Lean_Expr_const___override(x_1, x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_AC_buildNormProof_mkContext(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_9 = lean_array_get_size(x_2); +x_10 = lean_unsigned_to_nat(0u); +x_11 = lean_nat_dec_lt(x_10, x_9); +lean_dec(x_9); +if (x_11 == 0) { -lean_object* x_10; lean_object* x_11; uint8_t x_12; lean_object* x_13; size_t x_14; size_t x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_10 = lean_array_get_size(x_4); -x_11 = lean_unsigned_to_nat(0u); -x_12 = lean_nat_dec_lt(x_11, x_10); -lean_dec(x_10); -x_13 = lean_box(0); -x_14 = lean_array_size(x_4); -x_15 = 0; -x_16 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__3; -x_17 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__4; -x_18 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__7; -lean_inc(x_8); +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = l_Lean_instInhabitedExpr; +x_13 = l_outOfBounds___rarg(x_12); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_2); -lean_inc(x_1); -x_19 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1(x_1, x_2, x_3, x_13, x_16, x_17, x_18, x_14, x_15, x_4, x_5, x_6, x_7, x_8, x_9); -if (x_12 == 0) +x_14 = lean_infer_type(x_13, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_14) == 0) { -lean_dec(x_4); -if (lean_obj_tag(x_19) == 0) +lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_15); +x_17 = l_Lean_Meta_getLevel(x_15, x_4, x_5, x_6, x_7, x_16); +if (lean_obj_tag(x_17) == 0) { -lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; -x_185 = lean_ctor_get(x_19, 0); -lean_inc(x_185); -x_186 = lean_ctor_get(x_19, 1); -lean_inc(x_186); -lean_dec(x_19); -x_187 = l_Lean_instInhabitedExpr; -x_188 = l_outOfBounds___rarg(x_187); -x_20 = x_188; -x_21 = x_185; -x_22 = x_186; -goto block_184; +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); +lean_dec(x_17); +x_20 = l_Lean_Meta_AC_toACExpr___closed__4; +x_21 = l_Lean_Meta_AC_abstractAtoms_go(x_1, x_2, x_3, x_15, x_18, x_10, x_20, x_20, x_20, x_4, x_5, x_6, x_7, x_19); +return x_21; } else { -uint8_t x_189; -lean_dec(x_8); +uint8_t x_22; +lean_dec(x_15); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_189 = !lean_is_exclusive(x_19); -if (x_189 == 0) +x_22 = !lean_is_exclusive(x_17); +if (x_22 == 0) { -return x_19; +return x_17; } else { -lean_object* x_190; lean_object* x_191; lean_object* x_192; -x_190 = lean_ctor_get(x_19, 0); -x_191 = lean_ctor_get(x_19, 1); -lean_inc(x_191); -lean_inc(x_190); -lean_dec(x_19); -x_192 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_192, 0, x_190); -lean_ctor_set(x_192, 1, x_191); -return x_192; -} +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_17, 0); +x_24 = lean_ctor_get(x_17, 1); +lean_inc(x_24); +lean_inc(x_23); +lean_dec(x_17); +x_25 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +return x_25; } } -else -{ -if (lean_obj_tag(x_19) == 0) -{ -lean_object* x_193; lean_object* x_194; lean_object* x_195; -x_193 = lean_ctor_get(x_19, 0); -lean_inc(x_193); -x_194 = lean_ctor_get(x_19, 1); -lean_inc(x_194); -lean_dec(x_19); -x_195 = lean_array_fget(x_4, x_11); -lean_dec(x_4); -x_20 = x_195; -x_21 = x_193; -x_22 = x_194; -goto block_184; } else { -uint8_t x_196; -lean_dec(x_8); +uint8_t x_26; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -3986,948 +3999,1945 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_196 = !lean_is_exclusive(x_19); -if (x_196 == 0) +x_26 = !lean_is_exclusive(x_14); +if (x_26 == 0) { -return x_19; +return x_14; } else { -lean_object* x_197; lean_object* x_198; lean_object* x_199; -x_197 = lean_ctor_get(x_19, 0); -x_198 = lean_ctor_get(x_19, 1); -lean_inc(x_198); -lean_inc(x_197); -lean_dec(x_19); -x_199 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_199, 0, x_197); -lean_ctor_set(x_199, 1, x_198); -return x_199; +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_14, 0); +x_28 = lean_ctor_get(x_14, 1); +lean_inc(x_28); +lean_inc(x_27); +lean_dec(x_14); +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_27); +lean_ctor_set(x_29, 1, x_28); +return x_29; } } } -block_184: -{ -lean_object* x_23; uint8_t x_24; -x_23 = l_Array_unzip___rarg(x_21); -lean_dec(x_21); -x_24 = !lean_is_exclusive(x_23); -if (x_24 == 0) +else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_25 = lean_ctor_get(x_23, 0); -x_26 = lean_ctor_get(x_23, 1); -x_27 = lean_array_to_list(x_26); -x_28 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_28, 0, x_3); -lean_ctor_set(x_28, 1, x_13); -x_29 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__8; -lean_inc(x_28); -x_30 = l_Lean_Expr_const___override(x_29, x_28); -x_31 = lean_ctor_get(x_1, 1); -lean_inc(x_31); -lean_inc(x_31); -lean_inc(x_2); -x_32 = l_Lean_mkAppB(x_30, x_2, x_31); -x_33 = l_Lean_Meta_mkListLit(x_32, x_27, x_5, x_6, x_7, x_8, x_22); -if (lean_obj_tag(x_33) == 0) +lean_object* x_30; lean_object* x_31; +x_30 = lean_array_fget(x_2, x_10); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_31 = lean_infer_type(x_30, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_31) == 0) { -uint8_t x_34; -x_34 = !lean_is_exclusive(x_33); -if (x_34 == 0) +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_31, 0); +lean_inc(x_32); +x_33 = lean_ctor_get(x_31, 1); +lean_inc(x_33); +lean_dec(x_31); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_32); +x_34 = l_Lean_Meta_getLevel(x_32, x_4, x_5, x_6, x_7, x_33); +if (lean_obj_tag(x_34) == 0) { -lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_35 = lean_ctor_get(x_33, 0); -x_36 = l_Lean_Meta_AC_preContext___closed__6; -lean_inc(x_28); -x_37 = l_Lean_Expr_const___override(x_36, x_28); -lean_inc(x_31); -lean_inc(x_2); -x_38 = l_Lean_mkAppB(x_37, x_2, x_31); -x_39 = lean_ctor_get(x_1, 3); -lean_inc(x_39); -x_40 = l_Lean_Meta_AC_preContext___closed__8; -lean_inc(x_28); -x_41 = l_Lean_Expr_const___override(x_40, x_28); -lean_inc(x_31); -lean_inc(x_2); -x_42 = l_Lean_mkAppB(x_41, x_2, x_31); -x_43 = lean_ctor_get(x_1, 4); -lean_inc(x_43); -x_44 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__10; -x_45 = l_Lean_Expr_const___override(x_44, x_28); -if (lean_obj_tag(x_39) == 0) +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_35 = lean_ctor_get(x_34, 0); +lean_inc(x_35); +x_36 = lean_ctor_get(x_34, 1); +lean_inc(x_36); +lean_dec(x_34); +x_37 = l_Lean_Meta_AC_toACExpr___closed__4; +x_38 = l_Lean_Meta_AC_abstractAtoms_go(x_1, x_2, x_3, x_32, x_35, x_10, x_37, x_37, x_37, x_4, x_5, x_6, x_7, x_36); +return x_38; +} +else { -lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_46 = lean_ctor_get(x_1, 2); -lean_inc(x_46); +uint8_t x_39; +lean_dec(x_32); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); lean_dec(x_1); -x_47 = l_Lean_Expr_app___override(x_17, x_38); -x_48 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__11; -x_49 = l_Lean_Expr_app___override(x_48, x_47); -if (lean_obj_tag(x_43) == 0) +x_39 = !lean_is_exclusive(x_34); +if (x_39 == 0) { -lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_50 = l_Lean_Expr_app___override(x_17, x_42); -x_51 = l_Lean_Expr_app___override(x_48, x_50); -x_52 = l_Lean_mkApp7(x_45, x_2, x_31, x_46, x_49, x_51, x_35, x_20); -lean_ctor_set(x_23, 1, x_52); -lean_ctor_set(x_33, 0, x_23); -return x_33; +return x_34; } else { -lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; -x_53 = lean_ctor_get(x_43, 0); -lean_inc(x_53); -lean_dec(x_43); -lean_inc(x_42); -x_54 = l_Lean_Expr_app___override(x_17, x_42); -x_55 = l_Lean_mkAppB(x_18, x_42, x_53); -x_56 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__12; -x_57 = l_Lean_mkAppB(x_56, x_54, x_55); -x_58 = l_Lean_mkApp7(x_45, x_2, x_31, x_46, x_49, x_57, x_35, x_20); -lean_ctor_set(x_23, 1, x_58); -lean_ctor_set(x_33, 0, x_23); -return x_33; +lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_40 = lean_ctor_get(x_34, 0); +x_41 = lean_ctor_get(x_34, 1); +lean_inc(x_41); +lean_inc(x_40); +lean_dec(x_34); +x_42 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_42, 0, x_40); +lean_ctor_set(x_42, 1, x_41); +return x_42; +} } } else { -lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; -x_59 = lean_ctor_get(x_1, 2); -lean_inc(x_59); -lean_dec(x_1); -x_60 = lean_ctor_get(x_39, 0); -lean_inc(x_60); -lean_dec(x_39); -lean_inc(x_38); -x_61 = l_Lean_Expr_app___override(x_17, x_38); -x_62 = l_Lean_mkAppB(x_18, x_38, x_60); -x_63 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__12; -x_64 = l_Lean_mkAppB(x_63, x_61, x_62); -if (lean_obj_tag(x_43) == 0) -{ -lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_65 = l_Lean_Expr_app___override(x_17, x_42); -x_66 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__11; -x_67 = l_Lean_Expr_app___override(x_66, x_65); -x_68 = l_Lean_mkApp7(x_45, x_2, x_31, x_59, x_64, x_67, x_35, x_20); -lean_ctor_set(x_23, 1, x_68); -lean_ctor_set(x_33, 0, x_23); -return x_33; -} -else -{ -lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_69 = lean_ctor_get(x_43, 0); -lean_inc(x_69); -lean_dec(x_43); -lean_inc(x_42); -x_70 = l_Lean_Expr_app___override(x_17, x_42); -x_71 = l_Lean_mkAppB(x_18, x_42, x_69); -x_72 = l_Lean_mkAppB(x_63, x_70, x_71); -x_73 = l_Lean_mkApp7(x_45, x_2, x_31, x_59, x_64, x_72, x_35, x_20); -lean_ctor_set(x_23, 1, x_73); -lean_ctor_set(x_33, 0, x_23); -return x_33; -} -} -} -else -{ -lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; -x_74 = lean_ctor_get(x_33, 0); -x_75 = lean_ctor_get(x_33, 1); -lean_inc(x_75); -lean_inc(x_74); -lean_dec(x_33); -x_76 = l_Lean_Meta_AC_preContext___closed__6; -lean_inc(x_28); -x_77 = l_Lean_Expr_const___override(x_76, x_28); -lean_inc(x_31); -lean_inc(x_2); -x_78 = l_Lean_mkAppB(x_77, x_2, x_31); -x_79 = lean_ctor_get(x_1, 3); -lean_inc(x_79); -x_80 = l_Lean_Meta_AC_preContext___closed__8; -lean_inc(x_28); -x_81 = l_Lean_Expr_const___override(x_80, x_28); -lean_inc(x_31); -lean_inc(x_2); -x_82 = l_Lean_mkAppB(x_81, x_2, x_31); -x_83 = lean_ctor_get(x_1, 4); -lean_inc(x_83); -x_84 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__10; -x_85 = l_Lean_Expr_const___override(x_84, x_28); -if (lean_obj_tag(x_79) == 0) -{ -lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; -x_86 = lean_ctor_get(x_1, 2); -lean_inc(x_86); -lean_dec(x_1); -x_87 = l_Lean_Expr_app___override(x_17, x_78); -x_88 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__11; -x_89 = l_Lean_Expr_app___override(x_88, x_87); -if (lean_obj_tag(x_83) == 0) -{ -lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; -x_90 = l_Lean_Expr_app___override(x_17, x_82); -x_91 = l_Lean_Expr_app___override(x_88, x_90); -x_92 = l_Lean_mkApp7(x_85, x_2, x_31, x_86, x_89, x_91, x_74, x_20); -lean_ctor_set(x_23, 1, x_92); -x_93 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_93, 0, x_23); -lean_ctor_set(x_93, 1, x_75); -return x_93; -} -else -{ -lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; -x_94 = lean_ctor_get(x_83, 0); -lean_inc(x_94); -lean_dec(x_83); -lean_inc(x_82); -x_95 = l_Lean_Expr_app___override(x_17, x_82); -x_96 = l_Lean_mkAppB(x_18, x_82, x_94); -x_97 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__12; -x_98 = l_Lean_mkAppB(x_97, x_95, x_96); -x_99 = l_Lean_mkApp7(x_85, x_2, x_31, x_86, x_89, x_98, x_74, x_20); -lean_ctor_set(x_23, 1, x_99); -x_100 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_100, 0, x_23); -lean_ctor_set(x_100, 1, x_75); -return x_100; -} -} -else -{ -lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; -x_101 = lean_ctor_get(x_1, 2); -lean_inc(x_101); -lean_dec(x_1); -x_102 = lean_ctor_get(x_79, 0); -lean_inc(x_102); -lean_dec(x_79); -lean_inc(x_78); -x_103 = l_Lean_Expr_app___override(x_17, x_78); -x_104 = l_Lean_mkAppB(x_18, x_78, x_102); -x_105 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__12; -x_106 = l_Lean_mkAppB(x_105, x_103, x_104); -if (lean_obj_tag(x_83) == 0) -{ -lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; -x_107 = l_Lean_Expr_app___override(x_17, x_82); -x_108 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__11; -x_109 = l_Lean_Expr_app___override(x_108, x_107); -x_110 = l_Lean_mkApp7(x_85, x_2, x_31, x_101, x_106, x_109, x_74, x_20); -lean_ctor_set(x_23, 1, x_110); -x_111 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_111, 0, x_23); -lean_ctor_set(x_111, 1, x_75); -return x_111; -} -else -{ -lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; -x_112 = lean_ctor_get(x_83, 0); -lean_inc(x_112); -lean_dec(x_83); -lean_inc(x_82); -x_113 = l_Lean_Expr_app___override(x_17, x_82); -x_114 = l_Lean_mkAppB(x_18, x_82, x_112); -x_115 = l_Lean_mkAppB(x_105, x_113, x_114); -x_116 = l_Lean_mkApp7(x_85, x_2, x_31, x_101, x_106, x_115, x_74, x_20); -lean_ctor_set(x_23, 1, x_116); -x_117 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_117, 0, x_23); -lean_ctor_set(x_117, 1, x_75); -return x_117; -} -} -} -} -else -{ -uint8_t x_118; -lean_dec(x_31); -lean_dec(x_28); -lean_free_object(x_23); -lean_dec(x_25); -lean_dec(x_20); +uint8_t x_43; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_118 = !lean_is_exclusive(x_33); -if (x_118 == 0) -{ -return x_33; -} -else -{ -lean_object* x_119; lean_object* x_120; lean_object* x_121; -x_119 = lean_ctor_get(x_33, 0); -x_120 = lean_ctor_get(x_33, 1); -lean_inc(x_120); -lean_inc(x_119); -lean_dec(x_33); -x_121 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_121, 0, x_119); -lean_ctor_set(x_121, 1, x_120); -return x_121; -} -} -} -else -{ -lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; -x_122 = lean_ctor_get(x_23, 0); -x_123 = lean_ctor_get(x_23, 1); -lean_inc(x_123); -lean_inc(x_122); -lean_dec(x_23); -x_124 = lean_array_to_list(x_123); -x_125 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_125, 0, x_3); -lean_ctor_set(x_125, 1, x_13); -x_126 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__8; -lean_inc(x_125); -x_127 = l_Lean_Expr_const___override(x_126, x_125); -x_128 = lean_ctor_get(x_1, 1); -lean_inc(x_128); -lean_inc(x_128); -lean_inc(x_2); -x_129 = l_Lean_mkAppB(x_127, x_2, x_128); -x_130 = l_Lean_Meta_mkListLit(x_129, x_124, x_5, x_6, x_7, x_8, x_22); -if (lean_obj_tag(x_130) == 0) -{ -lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; -x_131 = lean_ctor_get(x_130, 0); -lean_inc(x_131); -x_132 = lean_ctor_get(x_130, 1); -lean_inc(x_132); -if (lean_is_exclusive(x_130)) { - lean_ctor_release(x_130, 0); - lean_ctor_release(x_130, 1); - x_133 = x_130; -} else { - lean_dec_ref(x_130); - x_133 = lean_box(0); -} -x_134 = l_Lean_Meta_AC_preContext___closed__6; -lean_inc(x_125); -x_135 = l_Lean_Expr_const___override(x_134, x_125); -lean_inc(x_128); -lean_inc(x_2); -x_136 = l_Lean_mkAppB(x_135, x_2, x_128); -x_137 = lean_ctor_get(x_1, 3); -lean_inc(x_137); -x_138 = l_Lean_Meta_AC_preContext___closed__8; -lean_inc(x_125); -x_139 = l_Lean_Expr_const___override(x_138, x_125); -lean_inc(x_128); -lean_inc(x_2); -x_140 = l_Lean_mkAppB(x_139, x_2, x_128); -x_141 = lean_ctor_get(x_1, 4); -lean_inc(x_141); -x_142 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__10; -x_143 = l_Lean_Expr_const___override(x_142, x_125); -if (lean_obj_tag(x_137) == 0) -{ -lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; -x_144 = lean_ctor_get(x_1, 2); -lean_inc(x_144); -lean_dec(x_1); -x_145 = l_Lean_Expr_app___override(x_17, x_136); -x_146 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__11; -x_147 = l_Lean_Expr_app___override(x_146, x_145); -if (lean_obj_tag(x_141) == 0) -{ -lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; -x_148 = l_Lean_Expr_app___override(x_17, x_140); -x_149 = l_Lean_Expr_app___override(x_146, x_148); -x_150 = l_Lean_mkApp7(x_143, x_2, x_128, x_144, x_147, x_149, x_131, x_20); -x_151 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_151, 0, x_122); -lean_ctor_set(x_151, 1, x_150); -if (lean_is_scalar(x_133)) { - x_152 = lean_alloc_ctor(0, 2, 0); -} else { - x_152 = x_133; -} -lean_ctor_set(x_152, 0, x_151); -lean_ctor_set(x_152, 1, x_132); -return x_152; -} -else +x_43 = !lean_is_exclusive(x_31); +if (x_43 == 0) { -lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; -x_153 = lean_ctor_get(x_141, 0); -lean_inc(x_153); -lean_dec(x_141); -lean_inc(x_140); -x_154 = l_Lean_Expr_app___override(x_17, x_140); -x_155 = l_Lean_mkAppB(x_18, x_140, x_153); -x_156 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__12; -x_157 = l_Lean_mkAppB(x_156, x_154, x_155); -x_158 = l_Lean_mkApp7(x_143, x_2, x_128, x_144, x_147, x_157, x_131, x_20); -x_159 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_159, 0, x_122); -lean_ctor_set(x_159, 1, x_158); -if (lean_is_scalar(x_133)) { - x_160 = lean_alloc_ctor(0, 2, 0); -} else { - x_160 = x_133; -} -lean_ctor_set(x_160, 0, x_159); -lean_ctor_set(x_160, 1, x_132); -return x_160; -} +return x_31; } else { -lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; -x_161 = lean_ctor_get(x_1, 2); -lean_inc(x_161); -lean_dec(x_1); -x_162 = lean_ctor_get(x_137, 0); -lean_inc(x_162); -lean_dec(x_137); -lean_inc(x_136); -x_163 = l_Lean_Expr_app___override(x_17, x_136); -x_164 = l_Lean_mkAppB(x_18, x_136, x_162); -x_165 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__12; -x_166 = l_Lean_mkAppB(x_165, x_163, x_164); -if (lean_obj_tag(x_141) == 0) -{ -lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; -x_167 = l_Lean_Expr_app___override(x_17, x_140); -x_168 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__11; -x_169 = l_Lean_Expr_app___override(x_168, x_167); -x_170 = l_Lean_mkApp7(x_143, x_2, x_128, x_161, x_166, x_169, x_131, x_20); -x_171 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_171, 0, x_122); -lean_ctor_set(x_171, 1, x_170); -if (lean_is_scalar(x_133)) { - x_172 = lean_alloc_ctor(0, 2, 0); -} else { - x_172 = x_133; -} -lean_ctor_set(x_172, 0, x_171); -lean_ctor_set(x_172, 1, x_132); -return x_172; +lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_44 = lean_ctor_get(x_31, 0); +x_45 = lean_ctor_get(x_31, 1); +lean_inc(x_45); +lean_inc(x_44); +lean_dec(x_31); +x_46 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_46, 0, x_44); +lean_ctor_set(x_46, 1, x_45); +return x_46; } -else -{ -lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; -x_173 = lean_ctor_get(x_141, 0); -lean_inc(x_173); -lean_dec(x_141); -lean_inc(x_140); -x_174 = l_Lean_Expr_app___override(x_17, x_140); -x_175 = l_Lean_mkAppB(x_18, x_140, x_173); -x_176 = l_Lean_mkAppB(x_165, x_174, x_175); -x_177 = l_Lean_mkApp7(x_143, x_2, x_128, x_161, x_166, x_176, x_131, x_20); -x_178 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_178, 0, x_122); -lean_ctor_set(x_178, 1, x_177); -if (lean_is_scalar(x_133)) { - x_179 = lean_alloc_ctor(0, 2, 0); -} else { - x_179 = x_133; } -lean_ctor_set(x_179, 0, x_178); -lean_ctor_set(x_179, 1, x_132); -return x_179; } } } -else +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1() { +_start: { -lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; -lean_dec(x_128); -lean_dec(x_125); -lean_dec(x_122); -lean_dec(x_20); -lean_dec(x_2); -lean_dec(x_1); -x_180 = lean_ctor_get(x_130, 0); -lean_inc(x_180); -x_181 = lean_ctor_get(x_130, 1); -lean_inc(x_181); -if (lean_is_exclusive(x_130)) { - lean_ctor_release(x_130, 0); - lean_ctor_release(x_130, 1); - x_182 = x_130; -} else { - lean_dec_ref(x_130); - x_182 = lean_box(0); -} -if (lean_is_scalar(x_182)) { - x_183 = lean_alloc_ctor(1, 2, 0); -} else { - x_183 = x_182; -} -lean_ctor_set(x_183, 0, x_180); -lean_ctor_set(x_183, 1, x_181); -return x_183; -} -} -} +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean", 4, 4); +return x_1; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__2() { _start: { -size_t x_16; size_t x_17; lean_object* x_18; -x_16 = lean_unbox_usize(x_8); -lean_dec(x_8); -x_17 = lean_unbox_usize(x_9); -lean_dec(x_9); -x_18 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_16, x_17, x_10, x_11, x_12, x_13, x_14, x_15); -return x_18; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Data", 4, 4); +return x_1; } } -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_convert___closed__1() { +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__3() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("Expr", 4, 4); +x_1 = lean_mk_string_unchecked("Variable", 8, 8); return x_1; } } -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_convert___closed__2() { +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__4() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("var", 3, 3); +x_1 = lean_mk_string_unchecked("mk", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_convert___closed__3() { +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__3; -x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__4; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1; +x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__2; x_3 = l_Lean_Meta_AC_getInstance___closed__2; -x_4 = l_Lean_Meta_AC_buildNormProof_convert___closed__1; -x_5 = l_Lean_Meta_AC_buildNormProof_convert___closed__2; +x_4 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__3; +x_5 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__4; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_convert___closed__4() { +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__6() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Meta_AC_buildNormProof_convert___closed__3; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Option", 6, 6); +return x_1; } } -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_convert___closed__5() { +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__7() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("op", 2, 2); +x_1 = lean_mk_string_unchecked("none", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_convert___closed__6() { +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__8() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__3; -x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__4; -x_3 = l_Lean_Meta_AC_getInstance___closed__2; -x_4 = l_Lean_Meta_AC_buildNormProof_convert___closed__1; -x_5 = l_Lean_Meta_AC_buildNormProof_convert___closed__5; -x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); -return x_6; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__6; +x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__7; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; } } -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_convert___closed__7() { +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__9() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("some", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Meta_AC_buildNormProof_convert___closed__6; -x_3 = l_Lean_Expr_const___override(x_2, x_1); +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__6; +x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__9; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Meta_AC_buildNormProof_convert(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, size_t x_8, size_t x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { -if (lean_obj_tag(x_1) == 0) +uint8_t x_16; +x_16 = lean_usize_dec_lt(x_9, x_8); +if (x_16 == 0) { -lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_2 = lean_ctor_get(x_1, 0); -lean_inc(x_2); +lean_object* x_17; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); lean_dec(x_1); -x_3 = l_Lean_mkNatLit(x_2); -x_4 = l_Lean_Meta_AC_buildNormProof_convert___closed__4; -x_5 = l_Lean_Expr_app___override(x_4, x_3); -return x_5; +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_10); +lean_ctor_set(x_17, 1, x_15); +return x_17; } else { -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_6 = lean_ctor_get(x_1, 0); +lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_18 = lean_array_uget(x_10, x_9); +x_19 = lean_unsigned_to_nat(0u); +x_20 = lean_array_uset(x_10, x_9, x_19); +x_21 = !lean_is_exclusive(x_18); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_22 = lean_ctor_get(x_18, 0); +x_23 = lean_ctor_get(x_18, 1); +lean_inc(x_4); +lean_inc(x_3); +lean_ctor_set_tag(x_18, 1); +lean_ctor_set(x_18, 1, x_4); +lean_ctor_set(x_18, 0, x_3); +x_24 = l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__2; +lean_inc(x_18); +x_25 = l_Lean_Expr_const___override(x_24, x_18); +x_26 = lean_ctor_get(x_1, 1); +lean_inc(x_26); +lean_inc(x_22); +lean_inc(x_26); +lean_inc(x_2); +x_27 = l_Lean_mkApp3(x_25, x_2, x_26, x_22); +x_28 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__5; +x_29 = l_Lean_Expr_const___override(x_28, x_18); +if (lean_obj_tag(x_23) == 0) +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; size_t x_35; size_t x_36; lean_object* x_37; +x_30 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__8; +lean_inc(x_5); +x_31 = l_Lean_Expr_const___override(x_30, x_5); lean_inc(x_6); -x_7 = lean_ctor_get(x_1, 1); -lean_inc(x_7); -lean_dec(x_1); -x_8 = l_Lean_Meta_AC_buildNormProof_convert(x_6); -x_9 = l_Lean_Meta_AC_buildNormProof_convert(x_7); -x_10 = l_Lean_Meta_AC_buildNormProof_convert___closed__7; -x_11 = l_Lean_mkAppB(x_10, x_8, x_9); -return x_11; -} -} +x_32 = l_Lean_Expr_app___override(x_6, x_27); +x_33 = l_Lean_Expr_app___override(x_31, x_32); +lean_inc(x_2); +x_34 = l_Lean_mkApp4(x_29, x_2, x_26, x_22, x_33); +x_35 = 1; +x_36 = lean_usize_add(x_9, x_35); +x_37 = lean_array_uset(x_20, x_9, x_34); +x_9 = x_36; +x_10 = x_37; +goto _start; } -LEAN_EXPORT lean_object* l_Lean_Meta_AC_buildNormProof_convertTarget(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: +else { -if (lean_obj_tag(x_3) == 0) +lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; size_t x_46; size_t x_47; lean_object* x_48; +x_39 = lean_ctor_get(x_23, 0); +lean_inc(x_39); +lean_dec(x_23); +x_40 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__10; +lean_inc(x_5); +x_41 = l_Lean_Expr_const___override(x_40, x_5); +lean_inc(x_27); +lean_inc(x_6); +x_42 = l_Lean_Expr_app___override(x_6, x_27); +lean_inc(x_7); +x_43 = l_Lean_mkAppB(x_7, x_27, x_39); +x_44 = l_Lean_mkAppB(x_41, x_42, x_43); +lean_inc(x_2); +x_45 = l_Lean_mkApp4(x_29, x_2, x_26, x_22, x_44); +x_46 = 1; +x_47 = lean_usize_add(x_9, x_46); +x_48 = lean_array_uset(x_20, x_9, x_45); +x_9 = x_47; +x_10 = x_48; +goto _start; +} +} +else { -lean_object* x_4; lean_object* x_5; uint8_t x_6; -lean_dec(x_1); -x_4 = lean_ctor_get(x_3, 0); -x_5 = lean_array_get_size(x_2); -x_6 = lean_nat_dec_lt(x_4, x_5); -lean_dec(x_5); -if (x_6 == 0) +lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; +x_50 = lean_ctor_get(x_18, 0); +x_51 = lean_ctor_get(x_18, 1); +lean_inc(x_51); +lean_inc(x_50); +lean_dec(x_18); +lean_inc(x_4); +lean_inc(x_3); +x_52 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_52, 0, x_3); +lean_ctor_set(x_52, 1, x_4); +x_53 = l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__2; +lean_inc(x_52); +x_54 = l_Lean_Expr_const___override(x_53, x_52); +x_55 = lean_ctor_get(x_1, 1); +lean_inc(x_55); +lean_inc(x_50); +lean_inc(x_55); +lean_inc(x_2); +x_56 = l_Lean_mkApp3(x_54, x_2, x_55, x_50); +x_57 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__5; +x_58 = l_Lean_Expr_const___override(x_57, x_52); +if (lean_obj_tag(x_51) == 0) { -lean_object* x_7; lean_object* x_8; -x_7 = l_Lean_instInhabitedExpr; -x_8 = l_outOfBounds___rarg(x_7); -return x_8; +lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; size_t x_64; size_t x_65; lean_object* x_66; +x_59 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__8; +lean_inc(x_5); +x_60 = l_Lean_Expr_const___override(x_59, x_5); +lean_inc(x_6); +x_61 = l_Lean_Expr_app___override(x_6, x_56); +x_62 = l_Lean_Expr_app___override(x_60, x_61); +lean_inc(x_2); +x_63 = l_Lean_mkApp4(x_58, x_2, x_55, x_50, x_62); +x_64 = 1; +x_65 = lean_usize_add(x_9, x_64); +x_66 = lean_array_uset(x_20, x_9, x_63); +x_9 = x_65; +x_10 = x_66; +goto _start; } else { -lean_object* x_9; -x_9 = lean_array_fget(x_2, x_4); -return x_9; +lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; size_t x_75; size_t x_76; lean_object* x_77; +x_68 = lean_ctor_get(x_51, 0); +lean_inc(x_68); +lean_dec(x_51); +x_69 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__10; +lean_inc(x_5); +x_70 = l_Lean_Expr_const___override(x_69, x_5); +lean_inc(x_56); +lean_inc(x_6); +x_71 = l_Lean_Expr_app___override(x_6, x_56); +lean_inc(x_7); +x_72 = l_Lean_mkAppB(x_7, x_56, x_68); +x_73 = l_Lean_mkAppB(x_70, x_71, x_72); +lean_inc(x_2); +x_74 = l_Lean_mkApp4(x_58, x_2, x_55, x_50, x_73); +x_75 = 1; +x_76 = lean_usize_add(x_9, x_75); +x_77 = lean_array_uset(x_20, x_9, x_74); +x_9 = x_76; +x_10 = x_77; +goto _start; } } -else -{ -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_10 = lean_ctor_get(x_3, 0); -x_11 = lean_ctor_get(x_3, 1); -x_12 = lean_ctor_get(x_1, 1); -lean_inc(x_12); -lean_inc(x_1); -x_13 = l_Lean_Meta_AC_buildNormProof_convertTarget(x_1, x_2, x_10); -x_14 = l_Lean_Meta_AC_buildNormProof_convertTarget(x_1, x_2, x_11); -x_15 = l_Lean_mkAppB(x_12, x_13, x_14); -return x_15; } } } -LEAN_EXPORT lean_object* l_Lean_Meta_AC_buildNormProof_convertTarget___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__1() { _start: { -lean_object* x_4; -x_4 = l_Lean_Meta_AC_buildNormProof_convertTarget(x_1, x_2, x_3); -lean_dec(x_3); -lean_dec(x_2); -return x_4; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_instInhabitedExpr; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__3(lean_object* x_1, lean_object* x_2) { +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__2() { _start: { -if (lean_obj_tag(x_2) == 0) +lean_object* x_1; +x_1 = lean_mk_string_unchecked("PLift", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__3() { +_start: { -lean_object* x_3; -x_3 = lean_box(0); +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__2; +x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } -else -{ -uint8_t x_4; -x_4 = !lean_is_exclusive(x_2); -if (x_4 == 0) -{ -lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; -x_5 = lean_ctor_get(x_2, 0); -x_6 = lean_ctor_get(x_2, 1); -x_7 = lean_ctor_get(x_1, 1); -x_8 = lean_array_get_size(x_7); -x_9 = lean_nat_dec_lt(x_5, x_8); -lean_dec(x_8); -if (x_9 == 0) -{ -uint8_t x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_10 = l_instInhabitedBool; -x_11 = lean_box(x_10); -x_12 = l_outOfBounds___rarg(x_11); -x_13 = lean_unbox(x_12); -lean_dec(x_12); -if (x_13 == 0) -{ -lean_object* x_14; -x_14 = l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__3(x_1, x_6); -lean_ctor_set(x_2, 1, x_14); -return x_2; } -else +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__4() { +_start: { -lean_free_object(x_2); -lean_dec(x_5); -x_2 = x_6; -goto _start; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = lean_box(0); +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; } } -else -{ -lean_object* x_16; uint8_t x_17; -x_16 = lean_array_fget(x_7, x_5); -x_17 = lean_unbox(x_16); -lean_dec(x_16); -if (x_17 == 0) +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__5() { +_start: { -lean_object* x_18; -x_18 = l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__3(x_1, x_6); -lean_ctor_set(x_2, 1, x_18); -return x_2; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__3; +x_2 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__4; +x_3 = l_Lean_Expr_const___override(x_1, x_2); +return x_3; } -else -{ -lean_free_object(x_2); -lean_dec(x_5); -x_2 = x_6; -goto _start; } +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("up", 2, 2); +return x_1; } } -else -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; -x_20 = lean_ctor_get(x_2, 0); -x_21 = lean_ctor_get(x_2, 1); -lean_inc(x_21); -lean_inc(x_20); -lean_dec(x_2); -x_22 = lean_ctor_get(x_1, 1); -x_23 = lean_array_get_size(x_22); -x_24 = lean_nat_dec_lt(x_20, x_23); -lean_dec(x_23); -if (x_24 == 0) -{ -uint8_t x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; -x_25 = l_instInhabitedBool; -x_26 = lean_box(x_25); -x_27 = l_outOfBounds___rarg(x_26); -x_28 = lean_unbox(x_27); -lean_dec(x_27); -if (x_28 == 0) +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__7() { +_start: { -lean_object* x_29; lean_object* x_30; -x_29 = l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__3(x_1, x_21); -x_30 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_30, 0, x_20); -lean_ctor_set(x_30, 1, x_29); -return x_30; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__2; +x_2 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__6; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; } -else +} +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__8() { +_start: { -lean_dec(x_20); -x_2 = x_21; -goto _start; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__7; +x_2 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__4; +x_3 = l_Lean_Expr_const___override(x_1, x_2); +return x_3; } } -else -{ -lean_object* x_32; uint8_t x_33; -x_32 = lean_array_fget(x_22, x_20); -x_33 = lean_unbox(x_32); -lean_dec(x_32); -if (x_33 == 0) +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__9() { +_start: { -lean_object* x_34; lean_object* x_35; -x_34 = l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__3(x_1, x_21); -x_35 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_35, 0, x_20); -lean_ctor_set(x_35, 1, x_34); -return x_35; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1; +x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__2; +x_3 = l_Lean_Meta_AC_getInstance___closed__2; +x_4 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__3; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; } -else +} +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__10() { +_start: { -lean_dec(x_20); -x_2 = x_21; -goto _start; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Context", 7, 7); +return x_1; } } +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__11() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1; +x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__2; +x_3 = l_Lean_Meta_AC_getInstance___closed__2; +x_4 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__10; +x_5 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__4; +x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); +return x_6; } } +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__12() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__8; +x_2 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__4; +x_3 = l_Lean_Expr_const___override(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Data_AC_removeNeutrals___at_Lean_Meta_AC_buildNormProof___spec__2(lean_object* x_1, lean_object* x_2) { +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__13() { _start: { -if (lean_obj_tag(x_2) == 0) -{ -lean_object* x_3; -x_3 = lean_box(0); +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__10; +x_2 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__4; +x_3 = l_Lean_Expr_const___override(x_1, x_2); return x_3; } +} +LEAN_EXPORT lean_object* l_Lean_Meta_AC_buildNormProof_mkContext(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; uint8_t x_12; lean_object* x_13; size_t x_14; size_t x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_10 = lean_array_get_size(x_4); +x_11 = lean_unsigned_to_nat(0u); +x_12 = lean_nat_dec_lt(x_11, x_10); +lean_dec(x_10); +x_13 = lean_box(0); +x_14 = lean_array_size(x_4); +x_15 = 0; +x_16 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__4; +x_17 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__5; +x_18 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__8; +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1(x_1, x_2, x_3, x_13, x_16, x_17, x_18, x_14, x_15, x_4, x_5, x_6, x_7, x_8, x_9); +if (x_12 == 0) +{ +lean_object* x_179; lean_object* x_180; +lean_dec(x_4); +x_179 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__1; +x_180 = l_outOfBounds___rarg(x_179); +x_20 = x_180; +goto block_178; +} +else +{ +lean_object* x_181; +x_181 = lean_array_fget(x_4, x_11); +lean_dec(x_4); +x_20 = x_181; +goto block_178; +} +block_178: +{ +uint8_t x_21; +x_21 = !lean_is_exclusive(x_19); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_22 = lean_ctor_get(x_19, 0); +x_23 = lean_ctor_get(x_19, 1); +x_24 = lean_ctor_get(x_20, 0); +lean_inc(x_24); +lean_dec(x_20); +x_25 = lean_array_to_list(x_22); +lean_ctor_set_tag(x_19, 1); +lean_ctor_set(x_19, 1, x_13); +lean_ctor_set(x_19, 0, x_3); +x_26 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__9; +lean_inc(x_19); +x_27 = l_Lean_Expr_const___override(x_26, x_19); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +lean_inc(x_28); +lean_inc(x_2); +x_29 = l_Lean_mkAppB(x_27, x_2, x_28); +x_30 = l_Lean_Meta_mkListLit(x_29, x_25, x_5, x_6, x_7, x_8, x_23); +if (lean_obj_tag(x_30) == 0) +{ +uint8_t x_31; +x_31 = !lean_is_exclusive(x_30); +if (x_31 == 0) +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_32 = lean_ctor_get(x_30, 0); +x_33 = l_Lean_Meta_AC_preContext___closed__6; +lean_inc(x_19); +x_34 = l_Lean_Expr_const___override(x_33, x_19); +lean_inc(x_28); +lean_inc(x_2); +x_35 = l_Lean_mkAppB(x_34, x_2, x_28); +x_36 = lean_ctor_get(x_1, 3); +lean_inc(x_36); +x_37 = l_Lean_Meta_AC_preContext___closed__8; +lean_inc(x_19); +x_38 = l_Lean_Expr_const___override(x_37, x_19); +lean_inc(x_28); +lean_inc(x_2); +x_39 = l_Lean_mkAppB(x_38, x_2, x_28); +x_40 = lean_ctor_get(x_1, 4); +lean_inc(x_40); +x_41 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__11; +x_42 = l_Lean_Expr_const___override(x_41, x_19); +if (lean_obj_tag(x_36) == 0) +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_43 = lean_ctor_get(x_1, 2); +lean_inc(x_43); +lean_dec(x_1); +x_44 = l_Lean_Expr_app___override(x_17, x_35); +x_45 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__12; +x_46 = l_Lean_Expr_app___override(x_45, x_44); +if (lean_obj_tag(x_40) == 0) +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_47 = l_Lean_Expr_app___override(x_17, x_39); +x_48 = l_Lean_Expr_app___override(x_45, x_47); +x_49 = l_Lean_mkApp7(x_42, x_2, x_28, x_43, x_46, x_48, x_32, x_24); +lean_ctor_set(x_30, 0, x_49); +return x_30; +} +else +{ +lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; +x_50 = lean_ctor_get(x_40, 0); +lean_inc(x_50); +lean_dec(x_40); +lean_inc(x_39); +x_51 = l_Lean_Expr_app___override(x_17, x_39); +x_52 = l_Lean_mkAppB(x_18, x_39, x_50); +x_53 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__13; +x_54 = l_Lean_mkAppB(x_53, x_51, x_52); +x_55 = l_Lean_mkApp7(x_42, x_2, x_28, x_43, x_46, x_54, x_32, x_24); +lean_ctor_set(x_30, 0, x_55); +return x_30; +} +} +else +{ +lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; +x_56 = lean_ctor_get(x_1, 2); +lean_inc(x_56); +lean_dec(x_1); +x_57 = lean_ctor_get(x_36, 0); +lean_inc(x_57); +lean_dec(x_36); +lean_inc(x_35); +x_58 = l_Lean_Expr_app___override(x_17, x_35); +x_59 = l_Lean_mkAppB(x_18, x_35, x_57); +x_60 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__13; +x_61 = l_Lean_mkAppB(x_60, x_58, x_59); +if (lean_obj_tag(x_40) == 0) +{ +lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_62 = l_Lean_Expr_app___override(x_17, x_39); +x_63 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__12; +x_64 = l_Lean_Expr_app___override(x_63, x_62); +x_65 = l_Lean_mkApp7(x_42, x_2, x_28, x_56, x_61, x_64, x_32, x_24); +lean_ctor_set(x_30, 0, x_65); +return x_30; +} +else +{ +lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; +x_66 = lean_ctor_get(x_40, 0); +lean_inc(x_66); +lean_dec(x_40); +lean_inc(x_39); +x_67 = l_Lean_Expr_app___override(x_17, x_39); +x_68 = l_Lean_mkAppB(x_18, x_39, x_66); +x_69 = l_Lean_mkAppB(x_60, x_67, x_68); +x_70 = l_Lean_mkApp7(x_42, x_2, x_28, x_56, x_61, x_69, x_32, x_24); +lean_ctor_set(x_30, 0, x_70); +return x_30; +} +} +} +else +{ +lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; +x_71 = lean_ctor_get(x_30, 0); +x_72 = lean_ctor_get(x_30, 1); +lean_inc(x_72); +lean_inc(x_71); +lean_dec(x_30); +x_73 = l_Lean_Meta_AC_preContext___closed__6; +lean_inc(x_19); +x_74 = l_Lean_Expr_const___override(x_73, x_19); +lean_inc(x_28); +lean_inc(x_2); +x_75 = l_Lean_mkAppB(x_74, x_2, x_28); +x_76 = lean_ctor_get(x_1, 3); +lean_inc(x_76); +x_77 = l_Lean_Meta_AC_preContext___closed__8; +lean_inc(x_19); +x_78 = l_Lean_Expr_const___override(x_77, x_19); +lean_inc(x_28); +lean_inc(x_2); +x_79 = l_Lean_mkAppB(x_78, x_2, x_28); +x_80 = lean_ctor_get(x_1, 4); +lean_inc(x_80); +x_81 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__11; +x_82 = l_Lean_Expr_const___override(x_81, x_19); +if (lean_obj_tag(x_76) == 0) +{ +lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; +x_83 = lean_ctor_get(x_1, 2); +lean_inc(x_83); +lean_dec(x_1); +x_84 = l_Lean_Expr_app___override(x_17, x_75); +x_85 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__12; +x_86 = l_Lean_Expr_app___override(x_85, x_84); +if (lean_obj_tag(x_80) == 0) +{ +lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; +x_87 = l_Lean_Expr_app___override(x_17, x_79); +x_88 = l_Lean_Expr_app___override(x_85, x_87); +x_89 = l_Lean_mkApp7(x_82, x_2, x_28, x_83, x_86, x_88, x_71, x_24); +x_90 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_90, 0, x_89); +lean_ctor_set(x_90, 1, x_72); +return x_90; +} +else +{ +lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; +x_91 = lean_ctor_get(x_80, 0); +lean_inc(x_91); +lean_dec(x_80); +lean_inc(x_79); +x_92 = l_Lean_Expr_app___override(x_17, x_79); +x_93 = l_Lean_mkAppB(x_18, x_79, x_91); +x_94 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__13; +x_95 = l_Lean_mkAppB(x_94, x_92, x_93); +x_96 = l_Lean_mkApp7(x_82, x_2, x_28, x_83, x_86, x_95, x_71, x_24); +x_97 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_97, 0, x_96); +lean_ctor_set(x_97, 1, x_72); +return x_97; +} +} +else +{ +lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; +x_98 = lean_ctor_get(x_1, 2); +lean_inc(x_98); +lean_dec(x_1); +x_99 = lean_ctor_get(x_76, 0); +lean_inc(x_99); +lean_dec(x_76); +lean_inc(x_75); +x_100 = l_Lean_Expr_app___override(x_17, x_75); +x_101 = l_Lean_mkAppB(x_18, x_75, x_99); +x_102 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__13; +x_103 = l_Lean_mkAppB(x_102, x_100, x_101); +if (lean_obj_tag(x_80) == 0) +{ +lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; +x_104 = l_Lean_Expr_app___override(x_17, x_79); +x_105 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__12; +x_106 = l_Lean_Expr_app___override(x_105, x_104); +x_107 = l_Lean_mkApp7(x_82, x_2, x_28, x_98, x_103, x_106, x_71, x_24); +x_108 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_108, 0, x_107); +lean_ctor_set(x_108, 1, x_72); +return x_108; +} +else +{ +lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; +x_109 = lean_ctor_get(x_80, 0); +lean_inc(x_109); +lean_dec(x_80); +lean_inc(x_79); +x_110 = l_Lean_Expr_app___override(x_17, x_79); +x_111 = l_Lean_mkAppB(x_18, x_79, x_109); +x_112 = l_Lean_mkAppB(x_102, x_110, x_111); +x_113 = l_Lean_mkApp7(x_82, x_2, x_28, x_98, x_103, x_112, x_71, x_24); +x_114 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_114, 0, x_113); +lean_ctor_set(x_114, 1, x_72); +return x_114; +} +} +} +} +else +{ +uint8_t x_115; +lean_dec(x_28); +lean_dec(x_19); +lean_dec(x_24); +lean_dec(x_2); +lean_dec(x_1); +x_115 = !lean_is_exclusive(x_30); +if (x_115 == 0) +{ +return x_30; +} +else +{ +lean_object* x_116; lean_object* x_117; lean_object* x_118; +x_116 = lean_ctor_get(x_30, 0); +x_117 = lean_ctor_get(x_30, 1); +lean_inc(x_117); +lean_inc(x_116); +lean_dec(x_30); +x_118 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_118, 0, x_116); +lean_ctor_set(x_118, 1, x_117); +return x_118; +} +} +} +else +{ +lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; +x_119 = lean_ctor_get(x_19, 0); +x_120 = lean_ctor_get(x_19, 1); +lean_inc(x_120); +lean_inc(x_119); +lean_dec(x_19); +x_121 = lean_ctor_get(x_20, 0); +lean_inc(x_121); +lean_dec(x_20); +x_122 = lean_array_to_list(x_119); +x_123 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_123, 0, x_3); +lean_ctor_set(x_123, 1, x_13); +x_124 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__9; +lean_inc(x_123); +x_125 = l_Lean_Expr_const___override(x_124, x_123); +x_126 = lean_ctor_get(x_1, 1); +lean_inc(x_126); +lean_inc(x_126); +lean_inc(x_2); +x_127 = l_Lean_mkAppB(x_125, x_2, x_126); +x_128 = l_Lean_Meta_mkListLit(x_127, x_122, x_5, x_6, x_7, x_8, x_120); +if (lean_obj_tag(x_128) == 0) +{ +lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; +x_129 = lean_ctor_get(x_128, 0); +lean_inc(x_129); +x_130 = lean_ctor_get(x_128, 1); +lean_inc(x_130); +if (lean_is_exclusive(x_128)) { + lean_ctor_release(x_128, 0); + lean_ctor_release(x_128, 1); + x_131 = x_128; +} else { + lean_dec_ref(x_128); + x_131 = lean_box(0); +} +x_132 = l_Lean_Meta_AC_preContext___closed__6; +lean_inc(x_123); +x_133 = l_Lean_Expr_const___override(x_132, x_123); +lean_inc(x_126); +lean_inc(x_2); +x_134 = l_Lean_mkAppB(x_133, x_2, x_126); +x_135 = lean_ctor_get(x_1, 3); +lean_inc(x_135); +x_136 = l_Lean_Meta_AC_preContext___closed__8; +lean_inc(x_123); +x_137 = l_Lean_Expr_const___override(x_136, x_123); +lean_inc(x_126); +lean_inc(x_2); +x_138 = l_Lean_mkAppB(x_137, x_2, x_126); +x_139 = lean_ctor_get(x_1, 4); +lean_inc(x_139); +x_140 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__11; +x_141 = l_Lean_Expr_const___override(x_140, x_123); +if (lean_obj_tag(x_135) == 0) +{ +lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; +x_142 = lean_ctor_get(x_1, 2); +lean_inc(x_142); +lean_dec(x_1); +x_143 = l_Lean_Expr_app___override(x_17, x_134); +x_144 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__12; +x_145 = l_Lean_Expr_app___override(x_144, x_143); +if (lean_obj_tag(x_139) == 0) +{ +lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; +x_146 = l_Lean_Expr_app___override(x_17, x_138); +x_147 = l_Lean_Expr_app___override(x_144, x_146); +x_148 = l_Lean_mkApp7(x_141, x_2, x_126, x_142, x_145, x_147, x_129, x_121); +if (lean_is_scalar(x_131)) { + x_149 = lean_alloc_ctor(0, 2, 0); +} else { + x_149 = x_131; +} +lean_ctor_set(x_149, 0, x_148); +lean_ctor_set(x_149, 1, x_130); +return x_149; +} +else +{ +lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; +x_150 = lean_ctor_get(x_139, 0); +lean_inc(x_150); +lean_dec(x_139); +lean_inc(x_138); +x_151 = l_Lean_Expr_app___override(x_17, x_138); +x_152 = l_Lean_mkAppB(x_18, x_138, x_150); +x_153 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__13; +x_154 = l_Lean_mkAppB(x_153, x_151, x_152); +x_155 = l_Lean_mkApp7(x_141, x_2, x_126, x_142, x_145, x_154, x_129, x_121); +if (lean_is_scalar(x_131)) { + x_156 = lean_alloc_ctor(0, 2, 0); +} else { + x_156 = x_131; +} +lean_ctor_set(x_156, 0, x_155); +lean_ctor_set(x_156, 1, x_130); +return x_156; +} +} +else +{ +lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; +x_157 = lean_ctor_get(x_1, 2); +lean_inc(x_157); +lean_dec(x_1); +x_158 = lean_ctor_get(x_135, 0); +lean_inc(x_158); +lean_dec(x_135); +lean_inc(x_134); +x_159 = l_Lean_Expr_app___override(x_17, x_134); +x_160 = l_Lean_mkAppB(x_18, x_134, x_158); +x_161 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__13; +x_162 = l_Lean_mkAppB(x_161, x_159, x_160); +if (lean_obj_tag(x_139) == 0) +{ +lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; +x_163 = l_Lean_Expr_app___override(x_17, x_138); +x_164 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__12; +x_165 = l_Lean_Expr_app___override(x_164, x_163); +x_166 = l_Lean_mkApp7(x_141, x_2, x_126, x_157, x_162, x_165, x_129, x_121); +if (lean_is_scalar(x_131)) { + x_167 = lean_alloc_ctor(0, 2, 0); +} else { + x_167 = x_131; +} +lean_ctor_set(x_167, 0, x_166); +lean_ctor_set(x_167, 1, x_130); +return x_167; +} +else +{ +lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; +x_168 = lean_ctor_get(x_139, 0); +lean_inc(x_168); +lean_dec(x_139); +lean_inc(x_138); +x_169 = l_Lean_Expr_app___override(x_17, x_138); +x_170 = l_Lean_mkAppB(x_18, x_138, x_168); +x_171 = l_Lean_mkAppB(x_161, x_169, x_170); +x_172 = l_Lean_mkApp7(x_141, x_2, x_126, x_157, x_162, x_171, x_129, x_121); +if (lean_is_scalar(x_131)) { + x_173 = lean_alloc_ctor(0, 2, 0); +} else { + x_173 = x_131; +} +lean_ctor_set(x_173, 0, x_172); +lean_ctor_set(x_173, 1, x_130); +return x_173; +} +} +} +else +{ +lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; +lean_dec(x_126); +lean_dec(x_123); +lean_dec(x_121); +lean_dec(x_2); +lean_dec(x_1); +x_174 = lean_ctor_get(x_128, 0); +lean_inc(x_174); +x_175 = lean_ctor_get(x_128, 1); +lean_inc(x_175); +if (lean_is_exclusive(x_128)) { + lean_ctor_release(x_128, 0); + lean_ctor_release(x_128, 1); + x_176 = x_128; +} else { + lean_dec_ref(x_128); + x_176 = lean_box(0); +} +if (lean_is_scalar(x_176)) { + x_177 = lean_alloc_ctor(1, 2, 0); +} else { + x_177 = x_176; +} +lean_ctor_set(x_177, 0, x_174); +lean_ctor_set(x_177, 1, x_175); +return x_177; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +_start: +{ +size_t x_16; size_t x_17; lean_object* x_18; +x_16 = lean_unbox_usize(x_8); +lean_dec(x_8); +x_17 = lean_unbox_usize(x_9); +lean_dec(x_9); +x_18 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_16, x_17, x_10, x_11, x_12, x_13, x_14, x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +return x_18; +} +} +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_convert___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Expr", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_convert___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("var", 3, 3); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_convert___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1; +x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__2; +x_3 = l_Lean_Meta_AC_getInstance___closed__2; +x_4 = l_Lean_Meta_AC_buildNormProof_convert___closed__1; +x_5 = l_Lean_Meta_AC_buildNormProof_convert___closed__2; +x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_convert___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_AC_buildNormProof_convert___closed__3; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_convert___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("op", 2, 2); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_convert___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1; +x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__2; +x_3 = l_Lean_Meta_AC_getInstance___closed__2; +x_4 = l_Lean_Meta_AC_buildNormProof_convert___closed__1; +x_5 = l_Lean_Meta_AC_buildNormProof_convert___closed__5; +x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_convert___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_AC_buildNormProof_convert___closed__6; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_AC_buildNormProof_convert(lean_object* x_1) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_2 = lean_ctor_get(x_1, 0); +lean_inc(x_2); +lean_dec(x_1); +x_3 = l_Lean_mkNatLit(x_2); +x_4 = l_Lean_Meta_AC_buildNormProof_convert___closed__4; +x_5 = l_Lean_Expr_app___override(x_4, x_3); +return x_5; +} +else +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +lean_dec(x_1); +x_8 = l_Lean_Meta_AC_buildNormProof_convert(x_6); +x_9 = l_Lean_Meta_AC_buildNormProof_convert(x_7); +x_10 = l_Lean_Meta_AC_buildNormProof_convert___closed__7; +x_11 = l_Lean_mkAppB(x_10, x_8, x_9); +return x_11; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_AC_buildNormProof_convertTarget(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +if (lean_obj_tag(x_3) == 0) +{ +lean_object* x_4; lean_object* x_5; uint8_t x_6; +lean_dec(x_1); +x_4 = lean_ctor_get(x_3, 0); +x_5 = lean_array_get_size(x_2); +x_6 = lean_nat_dec_lt(x_4, x_5); +lean_dec(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; +x_7 = l_Lean_instInhabitedExpr; +x_8 = l_outOfBounds___rarg(x_7); +return x_8; +} +else +{ +lean_object* x_9; +x_9 = lean_array_fget(x_2, x_4); +return x_9; +} +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_10 = lean_ctor_get(x_3, 0); +x_11 = lean_ctor_get(x_3, 1); +x_12 = lean_ctor_get(x_1, 1); +lean_inc(x_12); +lean_inc(x_1); +x_13 = l_Lean_Meta_AC_buildNormProof_convertTarget(x_1, x_2, x_10); +x_14 = l_Lean_Meta_AC_buildNormProof_convertTarget(x_1, x_2, x_11); +x_15 = l_Lean_mkAppB(x_12, x_13, x_14); +return x_15; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_AC_buildNormProof_convertTarget___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Lean_Meta_AC_buildNormProof_convertTarget(x_1, x_2, x_3); +lean_dec(x_3); +lean_dec(x_2); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof___spec__1(size_t x_1, size_t x_2, lean_object* x_3) { +_start: +{ +uint8_t x_4; +x_4 = lean_usize_dec_lt(x_2, x_1); +if (x_4 == 0) +{ +return x_3; +} +else +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; size_t x_9; size_t x_10; +x_5 = lean_array_uget(x_3, x_2); +x_6 = lean_unsigned_to_nat(0u); +x_7 = lean_array_uset(x_3, x_2, x_6); +x_8 = lean_ctor_get(x_5, 1); +lean_inc(x_8); +lean_dec(x_5); +x_9 = 1; +x_10 = lean_usize_add(x_2, x_9); +if (lean_obj_tag(x_8) == 0) +{ +uint8_t x_11; lean_object* x_12; lean_object* x_13; +x_11 = 0; +x_12 = lean_box(x_11); +x_13 = lean_array_uset(x_7, x_2, x_12); +x_2 = x_10; +x_3 = x_13; +goto _start; +} +else +{ +uint8_t x_15; lean_object* x_16; lean_object* x_17; +lean_dec(x_8); +x_15 = 1; +x_16 = lean_box(x_15); +x_17 = lean_array_uset(x_7, x_2, x_16); +x_2 = x_10; +x_3 = x_17; +goto _start; +} +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof___spec__2(size_t x_1, size_t x_2, lean_object* x_3) { +_start: +{ +uint8_t x_4; +x_4 = lean_usize_dec_lt(x_2, x_1); +if (x_4 == 0) +{ +return x_3; +} +else +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; size_t x_9; size_t x_10; lean_object* x_11; +x_5 = lean_array_uget(x_3, x_2); +x_6 = lean_unsigned_to_nat(0u); +x_7 = lean_array_uset(x_3, x_2, x_6); +x_8 = lean_ctor_get(x_5, 0); +lean_inc(x_8); +lean_dec(x_5); +x_9 = 1; +x_10 = lean_usize_add(x_2, x_9); +x_11 = lean_array_uset(x_7, x_2, x_8); +x_2 = x_10; +x_3 = x_11; +goto _start; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__5(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_3; +x_3 = lean_box(0); +return x_3; +} +else +{ +uint8_t x_4; +x_4 = !lean_is_exclusive(x_2); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; +x_5 = lean_ctor_get(x_2, 0); +x_6 = lean_ctor_get(x_2, 1); +x_7 = lean_ctor_get(x_1, 1); +x_8 = lean_array_get_size(x_7); +x_9 = lean_nat_dec_lt(x_5, x_8); +lean_dec(x_8); +if (x_9 == 0) +{ +uint8_t x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_10 = l_instInhabitedBool; +x_11 = lean_box(x_10); +x_12 = l_outOfBounds___rarg(x_11); +x_13 = lean_unbox(x_12); +lean_dec(x_12); +if (x_13 == 0) +{ +lean_object* x_14; +x_14 = l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__5(x_1, x_6); +lean_ctor_set(x_2, 1, x_14); +return x_2; +} +else +{ +lean_free_object(x_2); +lean_dec(x_5); +x_2 = x_6; +goto _start; +} +} +else +{ +lean_object* x_16; uint8_t x_17; +x_16 = lean_array_fget(x_7, x_5); +x_17 = lean_unbox(x_16); +lean_dec(x_16); +if (x_17 == 0) +{ +lean_object* x_18; +x_18 = l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__5(x_1, x_6); +lean_ctor_set(x_2, 1, x_18); +return x_2; +} +else +{ +lean_free_object(x_2); +lean_dec(x_5); +x_2 = x_6; +goto _start; +} +} +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; +x_20 = lean_ctor_get(x_2, 0); +x_21 = lean_ctor_get(x_2, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_2); +x_22 = lean_ctor_get(x_1, 1); +x_23 = lean_array_get_size(x_22); +x_24 = lean_nat_dec_lt(x_20, x_23); +lean_dec(x_23); +if (x_24 == 0) +{ +uint8_t x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; +x_25 = l_instInhabitedBool; +x_26 = lean_box(x_25); +x_27 = l_outOfBounds___rarg(x_26); +x_28 = lean_unbox(x_27); +lean_dec(x_27); +if (x_28 == 0) +{ +lean_object* x_29; lean_object* x_30; +x_29 = l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__5(x_1, x_21); +x_30 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_30, 0, x_20); +lean_ctor_set(x_30, 1, x_29); +return x_30; +} +else +{ +lean_dec(x_20); +x_2 = x_21; +goto _start; +} +} +else +{ +lean_object* x_32; uint8_t x_33; +x_32 = lean_array_fget(x_22, x_20); +x_33 = lean_unbox(x_32); +lean_dec(x_32); +if (x_33 == 0) +{ +lean_object* x_34; lean_object* x_35; +x_34 = l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__5(x_1, x_21); +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_20); +lean_ctor_set(x_35, 1, x_34); +return x_35; +} +else +{ +lean_dec(x_20); +x_2 = x_21; +goto _start; +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Data_AC_removeNeutrals___at_Lean_Meta_AC_buildNormProof___spec__4(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_3; +x_3 = lean_box(0); +return x_3; +} +else +{ +uint8_t x_4; +x_4 = !lean_is_exclusive(x_2); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +x_6 = l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__5(x_1, x_2); +if (lean_obj_tag(x_6) == 0) +{ +lean_object* x_7; lean_object* x_8; +x_7 = lean_box(0); +x_8 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_8, 0, x_5); +lean_ctor_set(x_8, 1, x_7); +return x_8; +} +else +{ +lean_dec(x_5); +return x_6; +} +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_9 = lean_ctor_get(x_2, 0); +x_10 = lean_ctor_get(x_2, 1); +lean_inc(x_10); +lean_inc(x_9); +lean_dec(x_2); +lean_inc(x_9); +x_11 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_11, 0, x_9); +lean_ctor_set(x_11, 1, x_10); +x_12 = l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__5(x_1, x_11); +if (lean_obj_tag(x_12) == 0) +{ +lean_object* x_13; lean_object* x_14; +x_13 = lean_box(0); +x_14 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_14, 0, x_9); +lean_ctor_set(x_14, 1, x_13); +return x_14; +} +else +{ +lean_dec(x_9); +return x_12; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Data_AC_norm___at_Lean_Meta_AC_buildNormProof___spec__3(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_3 = l_Lean_Data_AC_Expr_toList(x_2); +x_4 = l_Lean_Data_AC_removeNeutrals___at_Lean_Meta_AC_buildNormProof___spec__4(x_1, x_3); +x_5 = lean_ctor_get(x_1, 0); +x_6 = lean_ctor_get(x_5, 3); +if (lean_obj_tag(x_6) == 0) +{ +lean_object* x_7; +x_7 = lean_ctor_get(x_5, 4); +if (lean_obj_tag(x_7) == 0) +{ +return x_4; +} +else +{ +lean_object* x_8; +x_8 = l_Lean_Data_AC_mergeIdem(x_4); +return x_8; +} +} +else +{ +lean_object* x_9; +x_9 = lean_ctor_get(x_5, 4); +if (lean_obj_tag(x_9) == 0) +{ +lean_object* x_10; +x_10 = l_Lean_Data_AC_sort(x_4); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; +x_11 = l_Lean_Data_AC_sort(x_4); +x_12 = l_Lean_Data_AC_mergeIdem(x_11); +return x_12; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Data_AC_evalList___at_Lean_Meta_AC_buildNormProof___spec__6(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_3; +x_3 = l_Lean_Meta_AC_instEvalInformationPreContextACExpr___lambda__1___closed__1; +return x_3; +} +else +{ +lean_object* x_4; +x_4 = lean_ctor_get(x_2, 1); +lean_inc(x_4); +if (lean_obj_tag(x_4) == 0) +{ +lean_object* x_5; lean_object* x_6; +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +lean_dec(x_2); +x_6 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_6, 0, x_5); +return x_6; +} +else +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; +x_7 = lean_ctor_get(x_2, 0); +lean_inc(x_7); +lean_dec(x_2); +x_8 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_8, 0, x_7); +lean_inc(x_4); +x_9 = l_Lean_Data_AC_evalList___at_Lean_Meta_AC_buildNormProof___spec__6(x_1, x_4); +x_10 = !lean_is_exclusive(x_4); +if (x_10 == 0) +{ +lean_object* x_11; lean_object* x_12; +x_11 = lean_ctor_get(x_4, 1); +lean_dec(x_11); +x_12 = lean_ctor_get(x_4, 0); +lean_dec(x_12); +lean_ctor_set(x_4, 1, x_9); +lean_ctor_set(x_4, 0, x_8); +return x_4; +} +else +{ +lean_object* x_13; +lean_dec(x_4); +x_13 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_13, 0, x_8); +lean_ctor_set(x_13, 1, x_9); +return x_13; +} +} +} +} +} +static lean_object* _init_l_panic___at_Lean_Meta_AC_buildNormProof___spec__7___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Meta_instInhabitedMetaM___boxed), 5, 1); +lean_closure_set(x_1, 0, lean_box(0)); +return x_1; +} +} +LEAN_EXPORT lean_object* l_panic___at_Lean_Meta_AC_buildNormProof___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = l_panic___at_Lean_Meta_AC_buildNormProof___spec__7___closed__1; +x_8 = lean_panic_fn(x_7, x_1); +x_9 = lean_apply_5(x_8, x_2, x_3, x_4, x_5, x_6); +return x_9; +} +} +static lean_object* _init_l_Lean_Meta_AC_buildNormProof___lambda__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Bool", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_AC_buildNormProof___lambda__1___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("true", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_AC_buildNormProof___lambda__1___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Meta_AC_buildNormProof___lambda__1___closed__1; +x_2 = l_Lean_Meta_AC_buildNormProof___lambda__1___closed__2; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_AC_buildNormProof___lambda__1___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_AC_buildNormProof___lambda__1___closed__3; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_AC_buildNormProof___lambda__1___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("eq_of_norm", 10, 10); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_AC_buildNormProof___lambda__1___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1; +x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__2; +x_3 = l_Lean_Meta_AC_getInstance___closed__2; +x_4 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__10; +x_5 = l_Lean_Meta_AC_buildNormProof___lambda__1___closed__5; +x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_AC_buildNormProof___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_79; lean_object* x_80; uint8_t x_81; +x_79 = lean_array_get_size(x_3); +x_80 = lean_unsigned_to_nat(0u); +x_81 = lean_nat_dec_lt(x_80, x_79); +lean_dec(x_79); +if (x_81 == 0) +{ +lean_object* x_82; lean_object* x_83; +x_82 = l_Lean_instInhabitedExpr; +x_83 = l_outOfBounds___rarg(x_82); +x_10 = x_83; +goto block_78; +} +else +{ +lean_object* x_84; +x_84 = lean_array_fget(x_3, x_80); +x_10 = x_84; +goto block_78; +} +block_78: +{ +lean_object* x_11; +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_11 = lean_infer_type(x_10, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_11) == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_12); +x_14 = l_Lean_Meta_getLevel(x_12, x_5, x_6, x_7, x_8, x_13); +if (lean_obj_tag(x_14) == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_15); +lean_inc(x_12); +lean_inc(x_1); +x_17 = l_Lean_Meta_AC_buildNormProof_mkContext(x_1, x_12, x_15, x_4, x_5, x_6, x_7, x_8, x_16); +if (lean_obj_tag(x_17) == 0) +{ +lean_object* x_18; lean_object* x_19; size_t x_20; size_t x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); +lean_dec(x_17); +x_20 = lean_array_size(x_4); +x_21 = 0; +lean_inc(x_4); +x_22 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof___spec__1(x_20, x_21, x_4); +x_23 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof___spec__2(x_20, x_21, x_4); +lean_inc(x_1); +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_1); +lean_ctor_set(x_24, 1, x_22); +x_25 = l_Lean_Data_AC_norm___at_Lean_Meta_AC_buildNormProof___spec__3(x_24, x_2); +lean_dec(x_24); +x_26 = l_Lean_Data_AC_evalList___at_Lean_Meta_AC_buildNormProof___spec__6(x_1, x_25); +lean_inc(x_2); +x_27 = l_Lean_Meta_AC_buildNormProof_convert(x_2); +lean_inc(x_26); +x_28 = l_Lean_Meta_AC_buildNormProof_convert(x_26); +x_29 = lean_box(0); +x_30 = l_Lean_Meta_AC_buildNormProof___lambda__1___closed__4; +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_31 = l_Lean_Meta_mkEqRefl(x_30, x_5, x_6, x_7, x_8, x_19); +if (lean_obj_tag(x_31) == 0) +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_32 = lean_ctor_get(x_31, 0); +lean_inc(x_32); +x_33 = lean_ctor_get(x_31, 1); +lean_inc(x_33); +lean_dec(x_31); +x_34 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_34, 0, x_15); +lean_ctor_set(x_34, 1, x_29); +x_35 = l_Lean_Meta_AC_buildNormProof___lambda__1___closed__6; +x_36 = l_Lean_Expr_const___override(x_35, x_34); +x_37 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_32); +lean_ctor_set(x_37, 1, x_29); +x_38 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_38, 0, x_28); +lean_ctor_set(x_38, 1, x_37); +x_39 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_39, 0, x_27); +lean_ctor_set(x_39, 1, x_38); +x_40 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_40, 0, x_18); +lean_ctor_set(x_40, 1, x_39); +x_41 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_41, 0, x_12); +lean_ctor_set(x_41, 1, x_40); +x_42 = lean_array_mk(x_41); +x_43 = l_Lean_mkAppN(x_36, x_42); +lean_dec(x_42); +lean_inc(x_1); +x_44 = l_Lean_Meta_AC_buildNormProof_convertTarget(x_1, x_23, x_2); +lean_dec(x_2); +x_45 = l_Lean_Meta_AC_buildNormProof_convertTarget(x_1, x_23, x_26); +lean_dec(x_26); +lean_dec(x_23); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_46 = l_Lean_Meta_mkEq(x_44, x_45, x_5, x_6, x_7, x_8, x_33); +if (lean_obj_tag(x_46) == 0) +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_47 = lean_ctor_get(x_46, 0); +lean_inc(x_47); +x_48 = lean_ctor_get(x_46, 1); +lean_inc(x_48); +lean_dec(x_46); +x_49 = l_Lean_Meta_mkExpectedTypeHint(x_43, x_47, x_5, x_6, x_7, x_8, x_48); +if (lean_obj_tag(x_49) == 0) +{ +uint8_t x_50; +x_50 = !lean_is_exclusive(x_49); +if (x_50 == 0) +{ +return x_49; +} else { -uint8_t x_4; -x_4 = !lean_is_exclusive(x_2); -if (x_4 == 0) +lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_51 = lean_ctor_get(x_49, 0); +x_52 = lean_ctor_get(x_49, 1); +lean_inc(x_52); +lean_inc(x_51); +lean_dec(x_49); +x_53 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_53, 0, x_51); +lean_ctor_set(x_53, 1, x_52); +return x_53; +} +} +else { -lean_object* x_5; lean_object* x_6; -x_5 = lean_ctor_get(x_2, 0); -lean_inc(x_5); -x_6 = l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__3(x_1, x_2); -if (lean_obj_tag(x_6) == 0) +uint8_t x_54; +x_54 = !lean_is_exclusive(x_49); +if (x_54 == 0) { -lean_object* x_7; lean_object* x_8; -x_7 = lean_box(0); -x_8 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_8, 0, x_5); -lean_ctor_set(x_8, 1, x_7); -return x_8; +return x_49; } else { -lean_dec(x_5); -return x_6; +lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_55 = lean_ctor_get(x_49, 0); +x_56 = lean_ctor_get(x_49, 1); +lean_inc(x_56); +lean_inc(x_55); +lean_dec(x_49); +x_57 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_57, 0, x_55); +lean_ctor_set(x_57, 1, x_56); +return x_57; +} } } else { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_9 = lean_ctor_get(x_2, 0); -x_10 = lean_ctor_get(x_2, 1); -lean_inc(x_10); -lean_inc(x_9); -lean_dec(x_2); -lean_inc(x_9); -x_11 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_11, 0, x_9); -lean_ctor_set(x_11, 1, x_10); -x_12 = l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__3(x_1, x_11); -if (lean_obj_tag(x_12) == 0) +uint8_t x_58; +lean_dec(x_43); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_58 = !lean_is_exclusive(x_46); +if (x_58 == 0) { -lean_object* x_13; lean_object* x_14; -x_13 = lean_box(0); -x_14 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_14, 0, x_9); -lean_ctor_set(x_14, 1, x_13); -return x_14; +return x_46; } else { -lean_dec(x_9); -return x_12; -} -} +lean_object* x_59; lean_object* x_60; lean_object* x_61; +x_59 = lean_ctor_get(x_46, 0); +x_60 = lean_ctor_get(x_46, 1); +lean_inc(x_60); +lean_inc(x_59); +lean_dec(x_46); +x_61 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_61, 0, x_59); +lean_ctor_set(x_61, 1, x_60); +return x_61; } } } -LEAN_EXPORT lean_object* l_Lean_Data_AC_norm___at_Lean_Meta_AC_buildNormProof___spec__1(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_3 = l_Lean_Data_AC_Expr_toList(x_2); -x_4 = l_Lean_Data_AC_removeNeutrals___at_Lean_Meta_AC_buildNormProof___spec__2(x_1, x_3); -x_5 = lean_ctor_get(x_1, 0); -x_6 = lean_ctor_get(x_5, 3); -if (lean_obj_tag(x_6) == 0) +else { -lean_object* x_7; -x_7 = lean_ctor_get(x_5, 4); -if (lean_obj_tag(x_7) == 0) +uint8_t x_62; +lean_dec(x_28); +lean_dec(x_27); +lean_dec(x_26); +lean_dec(x_23); +lean_dec(x_18); +lean_dec(x_15); +lean_dec(x_12); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +lean_dec(x_1); +x_62 = !lean_is_exclusive(x_31); +if (x_62 == 0) { -return x_4; +return x_31; } else { -lean_object* x_8; -x_8 = l_Lean_Data_AC_mergeIdem(x_4); -return x_8; +lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_63 = lean_ctor_get(x_31, 0); +x_64 = lean_ctor_get(x_31, 1); +lean_inc(x_64); +lean_inc(x_63); +lean_dec(x_31); +x_65 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_65, 0, x_63); +lean_ctor_set(x_65, 1, x_64); +return x_65; +} } } else { -lean_object* x_9; -x_9 = lean_ctor_get(x_5, 4); -if (lean_obj_tag(x_9) == 0) +uint8_t x_66; +lean_dec(x_15); +lean_dec(x_12); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_66 = !lean_is_exclusive(x_17); +if (x_66 == 0) { -lean_object* x_10; -x_10 = l_Lean_Data_AC_sort(x_4); -return x_10; +return x_17; } else { -lean_object* x_11; lean_object* x_12; -x_11 = l_Lean_Data_AC_sort(x_4); -x_12 = l_Lean_Data_AC_mergeIdem(x_11); -return x_12; -} +lean_object* x_67; lean_object* x_68; lean_object* x_69; +x_67 = lean_ctor_get(x_17, 0); +x_68 = lean_ctor_get(x_17, 1); +lean_inc(x_68); +lean_inc(x_67); +lean_dec(x_17); +x_69 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_69, 0, x_67); +lean_ctor_set(x_69, 1, x_68); +return x_69; } } } -LEAN_EXPORT lean_object* l_Lean_Data_AC_evalList___at_Lean_Meta_AC_buildNormProof___spec__4(lean_object* x_1, lean_object* x_2) { -_start: +else { -if (lean_obj_tag(x_2) == 0) +uint8_t x_70; +lean_dec(x_12); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_70 = !lean_is_exclusive(x_14); +if (x_70 == 0) { -lean_object* x_3; -x_3 = l_Lean_Meta_AC_instEvalInformationPreContextACExpr___lambda__1___closed__1; -return x_3; +return x_14; } else { -lean_object* x_4; -x_4 = lean_ctor_get(x_2, 1); -lean_inc(x_4); -if (lean_obj_tag(x_4) == 0) -{ -lean_object* x_5; lean_object* x_6; -x_5 = lean_ctor_get(x_2, 0); -lean_inc(x_5); -lean_dec(x_2); -x_6 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_6, 0, x_5); -return x_6; +lean_object* x_71; lean_object* x_72; lean_object* x_73; +x_71 = lean_ctor_get(x_14, 0); +x_72 = lean_ctor_get(x_14, 1); +lean_inc(x_72); +lean_inc(x_71); +lean_dec(x_14); +x_73 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_73, 0, x_71); +lean_ctor_set(x_73, 1, x_72); +return x_73; +} +} } else { -lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; -x_7 = lean_ctor_get(x_2, 0); -lean_inc(x_7); +uint8_t x_74; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); lean_dec(x_2); -x_8 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_8, 0, x_7); -lean_inc(x_4); -x_9 = l_Lean_Data_AC_evalList___at_Lean_Meta_AC_buildNormProof___spec__4(x_1, x_4); -x_10 = !lean_is_exclusive(x_4); -if (x_10 == 0) +lean_dec(x_1); +x_74 = !lean_is_exclusive(x_11); +if (x_74 == 0) { -lean_object* x_11; lean_object* x_12; -x_11 = lean_ctor_get(x_4, 1); -lean_dec(x_11); -x_12 = lean_ctor_get(x_4, 0); -lean_dec(x_12); -lean_ctor_set(x_4, 1, x_9); -lean_ctor_set(x_4, 0, x_8); -return x_4; +return x_11; } else { -lean_object* x_13; -lean_dec(x_4); -x_13 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_13, 0, x_8); -lean_ctor_set(x_13, 1, x_9); -return x_13; +lean_object* x_75; lean_object* x_76; lean_object* x_77; +x_75 = lean_ctor_get(x_11, 0); +x_76 = lean_ctor_get(x_11, 1); +lean_inc(x_76); +lean_inc(x_75); +lean_dec(x_11); +x_77 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_77, 0, x_75); +lean_ctor_set(x_77, 1, x_76); +return x_77; } } } @@ -4937,43 +5947,41 @@ static lean_object* _init_l_Lean_Meta_AC_buildNormProof___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("Bool", 4, 4); +x_1 = lean_mk_string_unchecked("Eq", 2, 2); return x_1; } } static lean_object* _init_l_Lean_Meta_AC_buildNormProof___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("true", 4, 4); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_AC_buildNormProof___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } static lean_object* _init_l_Lean_Meta_AC_buildNormProof___closed__3() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_AC_buildNormProof___closed__1; -x_2 = l_Lean_Meta_AC_buildNormProof___closed__2; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean.Meta.Tactic.AC.Main", 24, 24); +return x_1; } } static lean_object* _init_l_Lean_Meta_AC_buildNormProof___closed__4() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Meta_AC_buildNormProof___closed__3; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean.Meta.AC.buildNormProof", 27, 27); +return x_1; } } static lean_object* _init_l_Lean_Meta_AC_buildNormProof___closed__5() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("eq_of_norm", 10, 10); +x_1 = lean_mk_string_unchecked("unexpected proof type", 21, 21); return x_1; } } @@ -4981,12 +5989,12 @@ static lean_object* _init_l_Lean_Meta_AC_buildNormProof___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__3; -x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__4; -x_3 = l_Lean_Meta_AC_getInstance___closed__2; -x_4 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__9; +x_1 = l_Lean_Meta_AC_buildNormProof___closed__3; +x_2 = l_Lean_Meta_AC_buildNormProof___closed__4; +x_3 = lean_unsigned_to_nat(129u); +x_4 = lean_unsigned_to_nat(52u); x_5 = l_Lean_Meta_AC_buildNormProof___closed__5; -x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); +x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; } } @@ -5003,51 +6011,29 @@ lean_inc(x_4); x_10 = l_Lean_Meta_AC_toACExpr(x_9, x_2, x_3, x_4, x_5, x_6, x_7, x_8); if (lean_obj_tag(x_10) == 0) { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_111; lean_object* x_112; uint8_t x_113; +lean_object* x_11; lean_object* x_12; uint8_t x_13; x_11 = lean_ctor_get(x_10, 0); lean_inc(x_11); x_12 = lean_ctor_get(x_10, 1); lean_inc(x_12); lean_dec(x_10); -x_13 = lean_ctor_get(x_11, 0); -lean_inc(x_13); -x_14 = lean_ctor_get(x_11, 1); -lean_inc(x_14); -if (lean_is_exclusive(x_11)) { - lean_ctor_release(x_11, 0); - lean_ctor_release(x_11, 1); - x_15 = x_11; -} else { - lean_dec_ref(x_11); - x_15 = lean_box(0); -} -x_111 = lean_array_get_size(x_13); -x_112 = lean_unsigned_to_nat(0u); -x_113 = lean_nat_dec_lt(x_112, x_111); -lean_dec(x_111); -if (x_113 == 0) -{ -lean_object* x_114; lean_object* x_115; -x_114 = l_Lean_instInhabitedExpr; -x_115 = l_outOfBounds___rarg(x_114); -x_16 = x_115; -goto block_110; -} -else -{ -lean_object* x_116; -x_116 = lean_array_fget(x_13, x_112); -x_16 = x_116; -goto block_110; -} -block_110: +x_13 = !lean_is_exclusive(x_11); +if (x_13 == 0) { -lean_object* x_17; +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_14 = lean_ctor_get(x_11, 0); +x_15 = lean_ctor_get(x_11, 1); +lean_inc(x_14); +lean_inc(x_1); +x_16 = lean_alloc_closure((void*)(l_Lean_Meta_AC_buildNormProof___lambda__1___boxed), 9, 3); +lean_closure_set(x_16, 0, x_1); +lean_closure_set(x_16, 1, x_15); +lean_closure_set(x_16, 2, x_14); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -x_17 = lean_infer_type(x_16, x_4, x_5, x_6, x_7, x_12); +x_17 = l_Lean_Meta_AC_abstractAtoms(x_1, x_14, x_16, x_4, x_5, x_6, x_7, x_12); if (lean_obj_tag(x_17) == 0) { lean_object* x_18; lean_object* x_19; lean_object* x_20; @@ -5060,439 +6046,384 @@ lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -lean_inc(x_18); -x_20 = l_Lean_Meta_getLevel(x_18, x_4, x_5, x_6, x_7, x_19); -if (lean_obj_tag(x_20) == 0) -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_20, 1); -lean_inc(x_22); -lean_dec(x_20); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_13); -lean_inc(x_21); -lean_inc(x_18); -lean_inc(x_1); -x_23 = l_Lean_Meta_AC_buildNormProof_mkContext(x_1, x_18, x_21, x_13, x_4, x_5, x_6, x_7, x_22); -if (lean_obj_tag(x_23) == 0) -{ -lean_object* x_24; lean_object* x_25; uint8_t x_26; -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_23, 1); -lean_inc(x_25); -lean_dec(x_23); -x_26 = !lean_is_exclusive(x_24); -if (x_26 == 0) -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_27 = lean_ctor_get(x_24, 0); -x_28 = lean_ctor_get(x_24, 1); -lean_inc(x_1); -lean_ctor_set(x_24, 1, x_27); -lean_ctor_set(x_24, 0, x_1); -x_29 = l_Lean_Data_AC_norm___at_Lean_Meta_AC_buildNormProof___spec__1(x_24, x_14); -lean_dec(x_24); -x_30 = l_Lean_Data_AC_evalList___at_Lean_Meta_AC_buildNormProof___spec__4(x_1, x_29); -x_31 = l_Lean_Meta_AC_buildNormProof_convertTarget(x_1, x_13, x_30); -lean_dec(x_13); -x_32 = l_Lean_Meta_AC_buildNormProof_convert(x_14); -x_33 = l_Lean_Meta_AC_buildNormProof_convert(x_30); -x_34 = lean_box(0); -x_35 = l_Lean_Meta_AC_buildNormProof___closed__4; -x_36 = l_Lean_Meta_mkEqRefl(x_35, x_4, x_5, x_6, x_7, x_25); -if (lean_obj_tag(x_36) == 0) +lean_inc(x_18); +x_20 = lean_infer_type(x_18, x_4, x_5, x_6, x_7, x_19); +if (lean_obj_tag(x_20) == 0) { -uint8_t x_37; -x_37 = !lean_is_exclusive(x_36); -if (x_37 == 0) +uint8_t x_21; +x_21 = !lean_is_exclusive(x_20); +if (x_21 == 0) { -lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_38 = lean_ctor_get(x_36, 0); -x_39 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_39, 0, x_21); -lean_ctor_set(x_39, 1, x_34); -x_40 = l_Lean_Meta_AC_buildNormProof___closed__6; -x_41 = l_Lean_Expr_const___override(x_40, x_39); -x_42 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_42, 0, x_38); -lean_ctor_set(x_42, 1, x_34); -x_43 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_43, 0, x_33); -lean_ctor_set(x_43, 1, x_42); -x_44 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_44, 0, x_32); -lean_ctor_set(x_44, 1, x_43); -x_45 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_45, 0, x_28); -lean_ctor_set(x_45, 1, x_44); -x_46 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_46, 0, x_18); -lean_ctor_set(x_46, 1, x_45); -x_47 = lean_array_mk(x_46); -x_48 = l_Lean_mkAppN(x_41, x_47); -lean_dec(x_47); -if (lean_is_scalar(x_15)) { - x_49 = lean_alloc_ctor(0, 2, 0); -} else { - x_49 = x_15; -} -lean_ctor_set(x_49, 0, x_48); -lean_ctor_set(x_49, 1, x_31); -lean_ctor_set(x_36, 0, x_49); -return x_36; +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; +x_22 = lean_ctor_get(x_20, 0); +x_23 = lean_ctor_get(x_20, 1); +x_24 = l_Lean_Meta_AC_buildNormProof___closed__2; +x_25 = lean_unsigned_to_nat(3u); +x_26 = l_Lean_Expr_isAppOfArity(x_22, x_24, x_25); +if (x_26 == 0) +{ +lean_object* x_27; lean_object* x_28; +lean_free_object(x_20); +lean_dec(x_22); +lean_dec(x_18); +lean_free_object(x_11); +x_27 = l_Lean_Meta_AC_buildNormProof___closed__6; +x_28 = l_panic___at_Lean_Meta_AC_buildNormProof___spec__7(x_27, x_4, x_5, x_6, x_7, x_23); +return x_28; } else { -lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; -x_50 = lean_ctor_get(x_36, 0); -x_51 = lean_ctor_get(x_36, 1); -lean_inc(x_51); -lean_inc(x_50); -lean_dec(x_36); -x_52 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_52, 0, x_21); -lean_ctor_set(x_52, 1, x_34); -x_53 = l_Lean_Meta_AC_buildNormProof___closed__6; -x_54 = l_Lean_Expr_const___override(x_53, x_52); -x_55 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_55, 0, x_50); -lean_ctor_set(x_55, 1, x_34); -x_56 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_56, 0, x_33); -lean_ctor_set(x_56, 1, x_55); -x_57 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_57, 0, x_32); -lean_ctor_set(x_57, 1, x_56); -x_58 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_58, 0, x_28); -lean_ctor_set(x_58, 1, x_57); -x_59 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_59, 0, x_18); -lean_ctor_set(x_59, 1, x_58); -x_60 = lean_array_mk(x_59); -x_61 = l_Lean_mkAppN(x_54, x_60); -lean_dec(x_60); -if (lean_is_scalar(x_15)) { - x_62 = lean_alloc_ctor(0, 2, 0); -} else { - x_62 = x_15; -} -lean_ctor_set(x_62, 0, x_61); -lean_ctor_set(x_62, 1, x_31); -x_63 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_63, 0, x_62); -lean_ctor_set(x_63, 1, x_51); -return x_63; +lean_object* x_29; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_29 = l_Lean_Expr_appArg_x21(x_22); +lean_dec(x_22); +lean_ctor_set(x_11, 1, x_29); +lean_ctor_set(x_11, 0, x_18); +lean_ctor_set(x_20, 0, x_11); +return x_20; } } else { -uint8_t x_64; -lean_dec(x_33); -lean_dec(x_32); -lean_dec(x_31); -lean_dec(x_28); -lean_dec(x_21); -lean_dec(x_18); -lean_dec(x_15); -x_64 = !lean_is_exclusive(x_36); -if (x_64 == 0) +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; +x_30 = lean_ctor_get(x_20, 0); +x_31 = lean_ctor_get(x_20, 1); +lean_inc(x_31); +lean_inc(x_30); +lean_dec(x_20); +x_32 = l_Lean_Meta_AC_buildNormProof___closed__2; +x_33 = lean_unsigned_to_nat(3u); +x_34 = l_Lean_Expr_isAppOfArity(x_30, x_32, x_33); +if (x_34 == 0) { +lean_object* x_35; lean_object* x_36; +lean_dec(x_30); +lean_dec(x_18); +lean_free_object(x_11); +x_35 = l_Lean_Meta_AC_buildNormProof___closed__6; +x_36 = l_panic___at_Lean_Meta_AC_buildNormProof___spec__7(x_35, x_4, x_5, x_6, x_7, x_31); return x_36; } else { -lean_object* x_65; lean_object* x_66; lean_object* x_67; -x_65 = lean_ctor_get(x_36, 0); -x_66 = lean_ctor_get(x_36, 1); -lean_inc(x_66); -lean_inc(x_65); -lean_dec(x_36); -x_67 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_67, 0, x_65); -lean_ctor_set(x_67, 1, x_66); -return x_67; +lean_object* x_37; lean_object* x_38; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_37 = l_Lean_Expr_appArg_x21(x_30); +lean_dec(x_30); +lean_ctor_set(x_11, 1, x_37); +lean_ctor_set(x_11, 0, x_18); +x_38 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_38, 0, x_11); +lean_ctor_set(x_38, 1, x_31); +return x_38; } } } else { -lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; -x_68 = lean_ctor_get(x_24, 0); -x_69 = lean_ctor_get(x_24, 1); -lean_inc(x_69); -lean_inc(x_68); -lean_dec(x_24); -lean_inc(x_1); -x_70 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_70, 0, x_1); -lean_ctor_set(x_70, 1, x_68); -x_71 = l_Lean_Data_AC_norm___at_Lean_Meta_AC_buildNormProof___spec__1(x_70, x_14); -lean_dec(x_70); -x_72 = l_Lean_Data_AC_evalList___at_Lean_Meta_AC_buildNormProof___spec__4(x_1, x_71); -x_73 = l_Lean_Meta_AC_buildNormProof_convertTarget(x_1, x_13, x_72); -lean_dec(x_13); -x_74 = l_Lean_Meta_AC_buildNormProof_convert(x_14); -x_75 = l_Lean_Meta_AC_buildNormProof_convert(x_72); -x_76 = lean_box(0); -x_77 = l_Lean_Meta_AC_buildNormProof___closed__4; -x_78 = l_Lean_Meta_mkEqRefl(x_77, x_4, x_5, x_6, x_7, x_25); -if (lean_obj_tag(x_78) == 0) +uint8_t x_39; +lean_dec(x_18); +lean_free_object(x_11); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_39 = !lean_is_exclusive(x_20); +if (x_39 == 0) { -lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; -x_79 = lean_ctor_get(x_78, 0); -lean_inc(x_79); -x_80 = lean_ctor_get(x_78, 1); -lean_inc(x_80); -if (lean_is_exclusive(x_78)) { - lean_ctor_release(x_78, 0); - lean_ctor_release(x_78, 1); - x_81 = x_78; -} else { - lean_dec_ref(x_78); - x_81 = lean_box(0); -} -x_82 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_82, 0, x_21); -lean_ctor_set(x_82, 1, x_76); -x_83 = l_Lean_Meta_AC_buildNormProof___closed__6; -x_84 = l_Lean_Expr_const___override(x_83, x_82); -x_85 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_85, 0, x_79); -lean_ctor_set(x_85, 1, x_76); -x_86 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_86, 0, x_75); -lean_ctor_set(x_86, 1, x_85); -x_87 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_87, 0, x_74); -lean_ctor_set(x_87, 1, x_86); -x_88 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_88, 0, x_69); -lean_ctor_set(x_88, 1, x_87); -x_89 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_89, 0, x_18); -lean_ctor_set(x_89, 1, x_88); -x_90 = lean_array_mk(x_89); -x_91 = l_Lean_mkAppN(x_84, x_90); -lean_dec(x_90); -if (lean_is_scalar(x_15)) { - x_92 = lean_alloc_ctor(0, 2, 0); -} else { - x_92 = x_15; -} -lean_ctor_set(x_92, 0, x_91); -lean_ctor_set(x_92, 1, x_73); -if (lean_is_scalar(x_81)) { - x_93 = lean_alloc_ctor(0, 2, 0); -} else { - x_93 = x_81; -} -lean_ctor_set(x_93, 0, x_92); -lean_ctor_set(x_93, 1, x_80); -return x_93; +return x_20; } else { -lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; -lean_dec(x_75); -lean_dec(x_74); -lean_dec(x_73); -lean_dec(x_69); -lean_dec(x_21); -lean_dec(x_18); -lean_dec(x_15); -x_94 = lean_ctor_get(x_78, 0); -lean_inc(x_94); -x_95 = lean_ctor_get(x_78, 1); -lean_inc(x_95); -if (lean_is_exclusive(x_78)) { - lean_ctor_release(x_78, 0); - lean_ctor_release(x_78, 1); - x_96 = x_78; -} else { - lean_dec_ref(x_78); - x_96 = lean_box(0); -} -if (lean_is_scalar(x_96)) { - x_97 = lean_alloc_ctor(1, 2, 0); -} else { - x_97 = x_96; -} -lean_ctor_set(x_97, 0, x_94); -lean_ctor_set(x_97, 1, x_95); -return x_97; +lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_40 = lean_ctor_get(x_20, 0); +x_41 = lean_ctor_get(x_20, 1); +lean_inc(x_41); +lean_inc(x_40); +lean_dec(x_20); +x_42 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_42, 0, x_40); +lean_ctor_set(x_42, 1, x_41); +return x_42; } } } else { -uint8_t x_98; -lean_dec(x_21); -lean_dec(x_18); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); +uint8_t x_43; +lean_free_object(x_11); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_1); -x_98 = !lean_is_exclusive(x_23); -if (x_98 == 0) +x_43 = !lean_is_exclusive(x_17); +if (x_43 == 0) { -return x_23; +return x_17; } else { -lean_object* x_99; lean_object* x_100; lean_object* x_101; -x_99 = lean_ctor_get(x_23, 0); -x_100 = lean_ctor_get(x_23, 1); -lean_inc(x_100); -lean_inc(x_99); -lean_dec(x_23); -x_101 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_101, 0, x_99); -lean_ctor_set(x_101, 1, x_100); -return x_101; +lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_44 = lean_ctor_get(x_17, 0); +x_45 = lean_ctor_get(x_17, 1); +lean_inc(x_45); +lean_inc(x_44); +lean_dec(x_17); +x_46 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_46, 0, x_44); +lean_ctor_set(x_46, 1, x_45); +return x_46; } } } else { -uint8_t x_102; -lean_dec(x_18); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_47 = lean_ctor_get(x_11, 0); +x_48 = lean_ctor_get(x_11, 1); +lean_inc(x_48); +lean_inc(x_47); +lean_dec(x_11); +lean_inc(x_47); +lean_inc(x_1); +x_49 = lean_alloc_closure((void*)(l_Lean_Meta_AC_buildNormProof___lambda__1___boxed), 9, 3); +lean_closure_set(x_49, 0, x_1); +lean_closure_set(x_49, 1, x_48); +lean_closure_set(x_49, 2, x_47); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_50 = l_Lean_Meta_AC_abstractAtoms(x_1, x_47, x_49, x_4, x_5, x_6, x_7, x_12); +if (lean_obj_tag(x_50) == 0) +{ +lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_51 = lean_ctor_get(x_50, 0); +lean_inc(x_51); +x_52 = lean_ctor_get(x_50, 1); +lean_inc(x_52); +lean_dec(x_50); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_51); +x_53 = lean_infer_type(x_51, x_4, x_5, x_6, x_7, x_52); +if (lean_obj_tag(x_53) == 0) +{ +lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; uint8_t x_59; +x_54 = lean_ctor_get(x_53, 0); +lean_inc(x_54); +x_55 = lean_ctor_get(x_53, 1); +lean_inc(x_55); +if (lean_is_exclusive(x_53)) { + lean_ctor_release(x_53, 0); + lean_ctor_release(x_53, 1); + x_56 = x_53; +} else { + lean_dec_ref(x_53); + x_56 = lean_box(0); +} +x_57 = l_Lean_Meta_AC_buildNormProof___closed__2; +x_58 = lean_unsigned_to_nat(3u); +x_59 = l_Lean_Expr_isAppOfArity(x_54, x_57, x_58); +if (x_59 == 0) +{ +lean_object* x_60; lean_object* x_61; +lean_dec(x_56); +lean_dec(x_54); +lean_dec(x_51); +x_60 = l_Lean_Meta_AC_buildNormProof___closed__6; +x_61 = l_panic___at_Lean_Meta_AC_buildNormProof___spec__7(x_60, x_4, x_5, x_6, x_7, x_55); +return x_61; +} +else +{ +lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_1); -x_102 = !lean_is_exclusive(x_20); -if (x_102 == 0) -{ -return x_20; +x_62 = l_Lean_Expr_appArg_x21(x_54); +lean_dec(x_54); +x_63 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_63, 0, x_51); +lean_ctor_set(x_63, 1, x_62); +if (lean_is_scalar(x_56)) { + x_64 = lean_alloc_ctor(0, 2, 0); +} else { + x_64 = x_56; +} +lean_ctor_set(x_64, 0, x_63); +lean_ctor_set(x_64, 1, x_55); +return x_64; +} } else { -lean_object* x_103; lean_object* x_104; lean_object* x_105; -x_103 = lean_ctor_get(x_20, 0); -x_104 = lean_ctor_get(x_20, 1); -lean_inc(x_104); -lean_inc(x_103); -lean_dec(x_20); -x_105 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_105, 0, x_103); -lean_ctor_set(x_105, 1, x_104); -return x_105; +lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; +lean_dec(x_51); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_65 = lean_ctor_get(x_53, 0); +lean_inc(x_65); +x_66 = lean_ctor_get(x_53, 1); +lean_inc(x_66); +if (lean_is_exclusive(x_53)) { + lean_ctor_release(x_53, 0); + lean_ctor_release(x_53, 1); + x_67 = x_53; +} else { + lean_dec_ref(x_53); + x_67 = lean_box(0); +} +if (lean_is_scalar(x_67)) { + x_68 = lean_alloc_ctor(1, 2, 0); +} else { + x_68 = x_67; } +lean_ctor_set(x_68, 0, x_65); +lean_ctor_set(x_68, 1, x_66); +return x_68; } } else { -uint8_t x_106; -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); +lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_1); -x_106 = !lean_is_exclusive(x_17); -if (x_106 == 0) -{ -return x_17; +x_69 = lean_ctor_get(x_50, 0); +lean_inc(x_69); +x_70 = lean_ctor_get(x_50, 1); +lean_inc(x_70); +if (lean_is_exclusive(x_50)) { + lean_ctor_release(x_50, 0); + lean_ctor_release(x_50, 1); + x_71 = x_50; +} else { + lean_dec_ref(x_50); + x_71 = lean_box(0); } -else -{ -lean_object* x_107; lean_object* x_108; lean_object* x_109; -x_107 = lean_ctor_get(x_17, 0); -x_108 = lean_ctor_get(x_17, 1); -lean_inc(x_108); -lean_inc(x_107); -lean_dec(x_17); -x_109 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_109, 0, x_107); -lean_ctor_set(x_109, 1, x_108); -return x_109; +if (lean_is_scalar(x_71)) { + x_72 = lean_alloc_ctor(1, 2, 0); +} else { + x_72 = x_71; } +lean_ctor_set(x_72, 0, x_69); +lean_ctor_set(x_72, 1, x_70); +return x_72; } } } else { -uint8_t x_117; +uint8_t x_73; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_1); -x_117 = !lean_is_exclusive(x_10); -if (x_117 == 0) +x_73 = !lean_is_exclusive(x_10); +if (x_73 == 0) { return x_10; } else { -lean_object* x_118; lean_object* x_119; lean_object* x_120; -x_118 = lean_ctor_get(x_10, 0); -x_119 = lean_ctor_get(x_10, 1); -lean_inc(x_119); -lean_inc(x_118); +lean_object* x_74; lean_object* x_75; lean_object* x_76; +x_74 = lean_ctor_get(x_10, 0); +x_75 = lean_ctor_get(x_10, 1); +lean_inc(x_75); +lean_inc(x_74); lean_dec(x_10); -x_120 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_120, 0, x_118); -lean_ctor_set(x_120, 1, x_119); -return x_120; +x_76 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_76, 0, x_74); +lean_ctor_set(x_76, 1, x_75); +return x_76; +} +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; size_t x_5; lean_object* x_6; +x_4 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof___spec__1(x_4, x_5, x_3); +return x_6; } } +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; size_t x_5; lean_object* x_6; +x_4 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof___spec__2(x_4, x_5, x_3); +return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__3___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__5___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__3(x_1, x_2); +x_3 = l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__5(x_1, x_2); lean_dec(x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Data_AC_removeNeutrals___at_Lean_Meta_AC_buildNormProof___spec__2___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Data_AC_removeNeutrals___at_Lean_Meta_AC_buildNormProof___spec__4___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Lean_Data_AC_removeNeutrals___at_Lean_Meta_AC_buildNormProof___spec__2(x_1, x_2); +x_3 = l_Lean_Data_AC_removeNeutrals___at_Lean_Meta_AC_buildNormProof___spec__4(x_1, x_2); lean_dec(x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Data_AC_norm___at_Lean_Meta_AC_buildNormProof___spec__1___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Data_AC_norm___at_Lean_Meta_AC_buildNormProof___spec__3___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Lean_Data_AC_norm___at_Lean_Meta_AC_buildNormProof___spec__1(x_1, x_2); +x_3 = l_Lean_Data_AC_norm___at_Lean_Meta_AC_buildNormProof___spec__3(x_1, x_2); lean_dec(x_2); lean_dec(x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Data_AC_evalList___at_Lean_Meta_AC_buildNormProof___spec__4___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Data_AC_evalList___at_Lean_Meta_AC_buildNormProof___spec__6___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Lean_Data_AC_evalList___at_Lean_Meta_AC_buildNormProof___spec__4(x_1, x_2); +x_3 = l_Lean_Data_AC_evalList___at_Lean_Meta_AC_buildNormProof___spec__6(x_1, x_2); lean_dec(x_1); return x_3; } } +LEAN_EXPORT lean_object* l_Lean_Meta_AC_buildNormProof___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l_Lean_Meta_AC_buildNormProof___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_3); +return x_10; +} +} LEAN_EXPORT lean_object* l_Lean_Meta_AC_post___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { @@ -7756,7 +8687,7 @@ static lean_object* _init_l___regBuiltin_Lean_Meta_AC_acRflTactic__1___closed__4 _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__3; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1; x_2 = l___regBuiltin_Lean_Meta_AC_acRflTactic__1___closed__1; x_3 = l___regBuiltin_Lean_Meta_AC_acRflTactic__1___closed__2; x_4 = l___regBuiltin_Lean_Meta_AC_acRflTactic__1___closed__3; @@ -7776,7 +8707,7 @@ static lean_object* _init_l___regBuiltin_Lean_Meta_AC_acRflTactic__1___closed__6 _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__3; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1; x_2 = l_Lean_Meta_AC_getInstance___closed__1; x_3 = l_Lean_Meta_AC_getInstance___closed__2; x_4 = l___regBuiltin_Lean_Meta_AC_acRflTactic__1___closed__5; @@ -9131,7 +10062,7 @@ static lean_object* _init_l_Lean_Meta_AC_evalNf0___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__3; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1; x_2 = l___regBuiltin_Lean_Meta_AC_acRflTactic__1___closed__1; x_3 = l___regBuiltin_Lean_Meta_AC_acRflTactic__1___closed__2; x_4 = l_Lean_Meta_AC_evalNf0___closed__1; @@ -9266,7 +10197,7 @@ static lean_object* _init_l___regBuiltin_Lean_Meta_AC_evalNf0__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__3; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1; x_2 = l_Lean_Meta_AC_getInstance___closed__1; x_3 = l_Lean_Meta_AC_getInstance___closed__2; x_4 = l___regBuiltin_Lean_Meta_AC_evalNf0__1___closed__1; @@ -9294,37 +10225,37 @@ x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); return x_6; } } -static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__1() { +static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__3; +x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__2() { +static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__1; +x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__1; x_2 = l_Lean_Meta_AC_getInstance___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__3() { +static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__2; +x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__2; x_2 = l_Lean_Meta_AC_getInstance___closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__4() { +static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__4() { _start: { lean_object* x_1; @@ -9332,17 +10263,17 @@ x_1 = lean_mk_string_unchecked("initFn", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__5() { +static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__3; -x_2 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__4; +x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__3; +x_2 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__4; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__6() { +static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__6() { _start: { lean_object* x_1; @@ -9350,57 +10281,57 @@ x_1 = lean_mk_string_unchecked("_@", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__7() { +static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__5; -x_2 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__6; +x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__5; +x_2 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__8() { +static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__7; -x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__3; +x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__7; +x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__9() { +static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__8; +x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__8; x_2 = l_Lean_Meta_AC_getInstance___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__10() { +static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__9; +x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__9; x_2 = l___regBuiltin_Lean_Meta_AC_acRflTactic__1___closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__11() { +static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__10; +x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__10; x_2 = l_Lean_Meta_AC_getInstance___closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__12() { +static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__12() { _start: { lean_object* x_1; @@ -9408,17 +10339,17 @@ x_1 = lean_mk_string_unchecked("Main", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__13() { +static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__11; -x_2 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__12; +x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__11; +x_2 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__12; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__14() { +static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__14() { _start: { lean_object* x_1; @@ -9426,33 +10357,33 @@ x_1 = lean_mk_string_unchecked("_hyg", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__15() { +static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__13; -x_2 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__14; +x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__13; +x_2 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__14; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__16() { +static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__16() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__15; -x_2 = lean_unsigned_to_nat(2895u); +x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__15; +x_2 = lean_unsigned_to_nat(6304u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304_(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; x_2 = l_Lean_Meta_AC_getInstance___closed__3; x_3 = 0; -x_4 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__16; +x_4 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__16; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); return x_5; } @@ -9560,6 +10491,18 @@ l_Lean_Meta_AC_toACExpr___closed__3 = _init_l_Lean_Meta_AC_toACExpr___closed__3( lean_mark_persistent(l_Lean_Meta_AC_toACExpr___closed__3); l_Lean_Meta_AC_toACExpr___closed__4 = _init_l_Lean_Meta_AC_toACExpr___closed__4(); lean_mark_persistent(l_Lean_Meta_AC_toACExpr___closed__4); +l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__1 = _init_l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__1); +l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__2 = _init_l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__2(); +lean_mark_persistent(l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__2); +l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__3 = _init_l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__3(); +lean_mark_persistent(l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__3); +l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__4 = _init_l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__4(); +lean_mark_persistent(l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__4); +l_Lean_Meta_AC_abstractAtoms_go___closed__1 = _init_l_Lean_Meta_AC_abstractAtoms_go___closed__1(); +lean_mark_persistent(l_Lean_Meta_AC_abstractAtoms_go___closed__1); +l_Lean_Meta_AC_abstractAtoms_go___closed__2 = _init_l_Lean_Meta_AC_abstractAtoms_go___closed__2(); +lean_mark_persistent(l_Lean_Meta_AC_abstractAtoms_go___closed__2); l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1 = _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1(); lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1); l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__2 = _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__2(); @@ -9580,10 +10523,6 @@ l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___cl lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__9); l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__10 = _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__10(); lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__10); -l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__11 = _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__11(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__11); -l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__12 = _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__12(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__12); l_Lean_Meta_AC_buildNormProof_mkContext___closed__1 = _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__1(); lean_mark_persistent(l_Lean_Meta_AC_buildNormProof_mkContext___closed__1); l_Lean_Meta_AC_buildNormProof_mkContext___closed__2 = _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__2(); @@ -9608,6 +10547,8 @@ l_Lean_Meta_AC_buildNormProof_mkContext___closed__11 = _init_l_Lean_Meta_AC_buil lean_mark_persistent(l_Lean_Meta_AC_buildNormProof_mkContext___closed__11); l_Lean_Meta_AC_buildNormProof_mkContext___closed__12 = _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__12(); lean_mark_persistent(l_Lean_Meta_AC_buildNormProof_mkContext___closed__12); +l_Lean_Meta_AC_buildNormProof_mkContext___closed__13 = _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__13(); +lean_mark_persistent(l_Lean_Meta_AC_buildNormProof_mkContext___closed__13); l_Lean_Meta_AC_buildNormProof_convert___closed__1 = _init_l_Lean_Meta_AC_buildNormProof_convert___closed__1(); lean_mark_persistent(l_Lean_Meta_AC_buildNormProof_convert___closed__1); l_Lean_Meta_AC_buildNormProof_convert___closed__2 = _init_l_Lean_Meta_AC_buildNormProof_convert___closed__2(); @@ -9622,6 +10563,20 @@ l_Lean_Meta_AC_buildNormProof_convert___closed__6 = _init_l_Lean_Meta_AC_buildNo lean_mark_persistent(l_Lean_Meta_AC_buildNormProof_convert___closed__6); l_Lean_Meta_AC_buildNormProof_convert___closed__7 = _init_l_Lean_Meta_AC_buildNormProof_convert___closed__7(); lean_mark_persistent(l_Lean_Meta_AC_buildNormProof_convert___closed__7); +l_panic___at_Lean_Meta_AC_buildNormProof___spec__7___closed__1 = _init_l_panic___at_Lean_Meta_AC_buildNormProof___spec__7___closed__1(); +lean_mark_persistent(l_panic___at_Lean_Meta_AC_buildNormProof___spec__7___closed__1); +l_Lean_Meta_AC_buildNormProof___lambda__1___closed__1 = _init_l_Lean_Meta_AC_buildNormProof___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Meta_AC_buildNormProof___lambda__1___closed__1); +l_Lean_Meta_AC_buildNormProof___lambda__1___closed__2 = _init_l_Lean_Meta_AC_buildNormProof___lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Meta_AC_buildNormProof___lambda__1___closed__2); +l_Lean_Meta_AC_buildNormProof___lambda__1___closed__3 = _init_l_Lean_Meta_AC_buildNormProof___lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Meta_AC_buildNormProof___lambda__1___closed__3); +l_Lean_Meta_AC_buildNormProof___lambda__1___closed__4 = _init_l_Lean_Meta_AC_buildNormProof___lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Meta_AC_buildNormProof___lambda__1___closed__4); +l_Lean_Meta_AC_buildNormProof___lambda__1___closed__5 = _init_l_Lean_Meta_AC_buildNormProof___lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Meta_AC_buildNormProof___lambda__1___closed__5); +l_Lean_Meta_AC_buildNormProof___lambda__1___closed__6 = _init_l_Lean_Meta_AC_buildNormProof___lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Meta_AC_buildNormProof___lambda__1___closed__6); l_Lean_Meta_AC_buildNormProof___closed__1 = _init_l_Lean_Meta_AC_buildNormProof___closed__1(); lean_mark_persistent(l_Lean_Meta_AC_buildNormProof___closed__1); l_Lean_Meta_AC_buildNormProof___closed__2 = _init_l_Lean_Meta_AC_buildNormProof___closed__2(); @@ -9720,39 +10675,39 @@ lean_mark_persistent(l___regBuiltin_Lean_Meta_AC_evalNf0__1___closed__3); if (builtin) {res = l___regBuiltin_Lean_Meta_AC_evalNf0__1(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__1 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__1(); -lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__1); -l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__2 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__2(); -lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__2); -l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__3 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__3(); -lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__3); -l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__4 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__4(); -lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__4); -l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__5 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__5(); -lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__5); -l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__6 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__6(); -lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__6); -l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__7 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__7(); -lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__7); -l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__8 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__8(); -lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__8); -l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__9 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__9(); -lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__9); -l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__10 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__10(); -lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__10); -l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__11 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__11(); -lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__11); -l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__12 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__12(); -lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__12); -l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__13 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__13(); -lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__13); -l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__14 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__14(); -lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__14); -l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__15 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__15(); -lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__15); -l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__16 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__16(); -lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__16); -if (builtin) {res = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895_(lean_io_mk_world()); +}l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__1 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__1(); +lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__1); +l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__2 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__2(); +lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__2); +l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__3 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__3(); +lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__3); +l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__4 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__4(); +lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__4); +l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__5 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__5(); +lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__5); +l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__6 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__6(); +lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__6); +l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__7 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__7(); +lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__7); +l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__8 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__8(); +lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__8); +l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__9 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__9(); +lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__9); +l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__10 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__10(); +lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__10); +l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__11 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__11(); +lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__11); +l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__12 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__12(); +lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__12); +l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__13 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__13(); +lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__13); +l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__14 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__14(); +lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__14); +l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__15 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__15(); +lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__15); +l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__16 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__16(); +lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__16); +if (builtin) {res = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }return lean_io_result_mk_ok(lean_box(0)); diff --git a/stage0/stdlib/Lean/Meta/Tactic/Backtrack.c b/stage0/stdlib/Lean/Meta/Tactic/Backtrack.c index 2b86a6dc16c7..39075f92a4a7 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Backtrack.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Backtrack.c @@ -27,6 +27,7 @@ lean_object* l_Lean_MVarId_getType___boxed(lean_object*, lean_object*, lean_obje LEAN_EXPORT lean_object* l_ReaderT_pure___at___private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run___spec__2(lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run___lambda__1___closed__4; static lean_object* l___private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run___lambda__10___closed__1; +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at___private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_processIndependentGoals___spec__7(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_processIndependentGoals___lambda__1___closed__6; static lean_object* l___private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_processIndependentGoals___lambda__4___closed__2; double lean_float_div(double, double); @@ -68,7 +69,6 @@ static lean_object* l___private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_B LEAN_EXPORT lean_object* l_Lean_withTraceNode___at___private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run___spec__6___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_ReaderT_pure___at___private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_bindTR_go___at___private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_processIndependentGoals___spec__7(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterMapTR_go___at_Lean_Meta_Tactic_Backtrack_Backtrack_tryAllM___spec__2(lean_object*, lean_object*); lean_object* l_List_appendTR___rarg(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run___lambda__1___closed__3; @@ -5553,7 +5553,7 @@ return x_26; } } } -LEAN_EXPORT lean_object* l_List_bindTR_go___at___private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_processIndependentGoals___spec__7(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at___private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_processIndependentGoals___spec__7(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -6418,7 +6418,7 @@ lean_inc(x_19); x_20 = lean_ctor_get(x_17, 1); lean_inc(x_20); lean_dec(x_17); -x_21 = l_List_bindTR_go___at___private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_processIndependentGoals___spec__7(x_20, x_3); +x_21 = l_List_flatMapTR_go___at___private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_processIndependentGoals___spec__7(x_20, x_3); lean_inc(x_4); lean_inc(x_21); lean_inc(x_19); diff --git a/stage0/stdlib/Lean/Meta/Tactic/Cases.c b/stage0/stdlib/Lean/Meta/Tactic/Cases.c index 95c82dff9dff..ac7fa2be1cd0 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Cases.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Cases.c @@ -223,6 +223,7 @@ lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_hasIndepIndices___spec__44(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_hasIndepIndices___spec__14(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_hasIndepIndices___spec__10(lean_object*, lean_object*, lean_object*, size_t, size_t); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_toCasesSubgoals___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_hasIndepIndices___spec__52(lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_hasIndepIndices___spec__20___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_forInAux___at_Lean_MVarId_casesRec___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -300,7 +301,6 @@ lean_object* l_Array_extract___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_withNewEqs___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_exactlyOne(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_MVarId_casesRec___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_toCasesSubgoals___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Cases_cases___closed__1; lean_object* l_Lean_Meta_introNCore(lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_Cases___hyg_3709____closed__12; @@ -375,6 +375,7 @@ lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_SynthInstance_0_ LEAN_EXPORT lean_object* l_Lean_PersistentArray_forInAux___at_Lean_MVarId_casesRec___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Cases_cases___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_generalizeIndices___spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_toCasesSubgoals___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_MVarId_casesRec___spec__1(lean_object*, lean_object*); uint8_t l_Lean_Expr_hasFVar(lean_object*); @@ -393,7 +394,6 @@ lean_object* l_Lean_addTrace___at_Lean_Meta_processPostponed_loop___spec__2(lean LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_generalizeIndices___spec__1___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_throwInductiveTypeExpected___spec__1(lean_object*); static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_Cases___hyg_3709____closed__4; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_toCasesSubgoals___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_hasIndepIndices___spec__49(lean_object*, lean_object*, lean_object*, size_t, size_t); lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Cases_cases___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -12595,7 +12595,7 @@ lean_dec(x_1); return x_8; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_toCasesSubgoals___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_toCasesSubgoals___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; uint8_t x_12; @@ -12749,15 +12749,15 @@ lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; x_6 = lean_array_get_size(x_1); x_7 = lean_mk_empty_array_with_capacity(x_6); x_8 = lean_unsigned_to_nat(0u); -x_9 = l_Array_mapIdxM_map___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_toCasesSubgoals___spec__1(x_1, x_2, x_3, x_4, x_5, x_1, x_6, x_8, lean_box(0), x_7); +x_9 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_toCasesSubgoals___spec__1(x_1, x_2, x_3, x_4, x_5, x_1, x_6, x_8, lean_box(0), x_7); return x_9; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_toCasesSubgoals___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_toCasesSubgoals___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; -x_11 = l_Array_mapIdxM_map___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_toCasesSubgoals___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_toCasesSubgoals___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_6); lean_dec(x_5); lean_dec(x_2); diff --git a/stage0/stdlib/Lean/Meta/Tactic/FunInd.c b/stage0/stdlib/Lean/Meta/Tactic/FunInd.c index 5e6a7ee4e351..d88a1bea6ff1 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/FunInd.c +++ b/stage0/stdlib/Lean/Meta/Tactic/FunInd.c @@ -38,10 +38,10 @@ static lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Tactic_FunInd_buil LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_buildInductionCase___closed__7; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__16___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__17___lambda__2___closed__2; +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__17___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_buildInductionBody___spec__26(lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_cleanPackedArgs___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__5; LEAN_EXPORT lean_object* l_StateT_bind___at_Lean_Tactic_FunInd_buildInductionBody___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Tactic_FunInd_buildInductionBody___spec__6___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_ArgsPacker_curryParam___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -55,15 +55,14 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_derive LEAN_EXPORT lean_object* l_Lean_getConstInfo___at_Lean_Tactic_FunInd_buildInductionBody___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_MatcherApp_withUserNames___at_Lean_Tactic_FunInd_buildInductionBody___spec__37(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_foldAndCollect___spec__25___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__22(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__22(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Expr_withAppAux___at_Lean_Tactic_FunInd_unpackMutualInduction___spec__1___lambda__2___closed__4; -LEAN_EXPORT lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616_(lean_object*); lean_object* l_Lean_getConstInfo___at_Lean_Meta_mkConstWithFreshMVarLevels___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_MatcherApp_transform___at_Lean_Tactic_FunInd_buildInductionBody___spec__29___closed__3; +LEAN_EXPORT lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__22___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_cleanPackedArgs___lambda__5___closed__5; static lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__10___closed__1; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_withLetDecl___at___private_Lean_Meta_Tactic_Simp_SimpTheorems_0__Lean_Meta_isPerm___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); lean_object* l_Lean_mkAppN(lean_object*, lean_object*); @@ -71,21 +70,17 @@ static lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__4__ static lean_object* l_Lean_getConstInfo___at_Lean_Tactic_FunInd_foldAndCollect___spec__3___closed__3; static lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__13___closed__4; extern lean_object* l_Lean_Elab_WF_instInhabitedEqnInfo; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_buildInductionBody___spec__38(lean_object*, size_t, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkPProdFst(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Tactic_FunInd_foldAndCollect___spec__6___closed__3; lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_buildInductionBody___spec__17(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_MatcherApp_transform___at_Lean_Tactic_FunInd_buildInductionBody___spec__29___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Structural_Positions_mapMwith___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__12___closed__1; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____closed__2; LEAN_EXPORT uint8_t l_Lean_logAt___at_Lean_Tactic_FunInd_buildInductionBody___spec__41___lambda__2(lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__26___closed__2; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_cleanupAfter_go___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_qsort_sort___at_Lean_Elab_Structural_Positions_groupAndSort___spec__3(lean_object*, lean_object*, lean_object*); @@ -147,22 +142,23 @@ uint8_t l_Lean_Expr_isAppOfArity(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Tactic_FunInd_foldAndCollect___spec__9___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__24(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_MatcherApp_withUserNames___at_Lean_Meta_MatcherApp_inferMatchType___spec__10___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__8___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_StateT_pure___at_Lean_Tactic_FunInd_buildInductionBody___spec__46___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isApp(lean_object*); +static lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__20___closed__2; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__19___lambda__3___boxed(lean_object**); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__11(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_buildInductionCase___closed__6; +static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__10; lean_object* l_Array_findIdx_x3f_loop___rarg(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_sort___override(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_buildInductionBody___spec__43___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_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__16___lambda__2___closed__2; lean_object* l_Lean_MessageData_ofList(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__16___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__17___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__23(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__23(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PersistentArray_push___rarg(lean_object*, lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_mkFreshFVarId___at_Lean_Tactic_FunInd_buildInductionBody___spec__22(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -171,10 +167,9 @@ lean_object* l_Array_toSubarray___rarg(lean_object*, lean_object*, lean_object*) static lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Tactic_FunInd_foldAndCollect___spec__1___lambda__3___closed__1; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__12___boxed(lean_object**); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -uint8_t l_Array_contains___at_Lean_findField_x3f___spec__1(lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__16___lambda__4___closed__3; -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__4(lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__1; static lean_object* l_Lean_logAt___at_Lean_Tactic_FunInd_buildInductionBody___spec__41___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -196,7 +191,6 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_buildI static lean_object* l_Lean_Tactic_FunInd_deriveInduction___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__10___boxed(lean_object**); lean_object* l_Lean_Expr_mdata___override(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_buildInductionBody___spec__19___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_cleanupAfter_cleanupAfter_x3f___spec__5(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Structural_getRecArgInfo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -220,7 +214,6 @@ lean_object* l_Lean_Meta_forallTelescope___at_Lean_Meta_mapForallTelescope_x27__ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_buildInductionBody___spec__35___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_deriveInduction___lambda__1___closed__2; extern lean_object* l_Lean_casesOnSuffix; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getTailPos_x3f(lean_object*, uint8_t); lean_object* l_Lean_Meta_Match_MatcherInfo_arity(lean_object*); lean_object* l_Lean_ConstantInfo_name(lean_object*); @@ -238,7 +231,6 @@ static lean_object* l_Lean_Tactic_FunInd_abstractIndependentMVars___closed__3; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_buildInductionBody___spec__24(lean_object*); lean_object* l_Lean_Expr_fvarId_x21(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Structural_Positions_mapMwith___at_Lean_Tactic_FunInd_deriveInductionStructural___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_Lean_Tactic_FunInd_buildInductionBody___lambda__26___closed__1; LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Tactic_FunInd_buildInductionCase___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_panic___at_Lean_Tactic_FunInd_buildInductionBody___spec__13___closed__1; static lean_object* l_Lean_Expr_withAppAux___at_Lean_Tactic_FunInd_unpackMutualInduction___spec__1___lambda__3___closed__2; @@ -259,12 +251,12 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_foldAndCollec LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInduction___lambda__2(lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___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_Lean_Meta_forallTelescope___at_Lean_Tactic_FunInd_deriveUnaryInduction___spec__3(lean_object*); +static lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__17___closed__1; lean_object* l_Lean_Meta_forallTelescopeReducing___at_Lean_Meta_getParamNames___spec__2___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_hasSyntheticSorry(lean_object*); static lean_object* l_Lean_Expr_withAppAux___at_Lean_Tactic_FunInd_unpackMutualInduction___spec__1___lambda__2___closed__2; static lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___closed__1; LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at_Lean_Tactic_FunInd_mkLambdaFVarsMasked___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__10; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__4___boxed(lean_object**); static lean_object* l_Lean_Tactic_FunInd_deriveInduction___closed__1; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_foldAndCollect___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -278,7 +270,6 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_buildInd LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_assertIHs___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__18(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_elimOptParam___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__10; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_cleanupAfter_cleanupAfter_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Nat_nextPowerOfTwo_go(lean_object*, lean_object*, lean_object*); lean_object* l_List_get___rarg(lean_object*, lean_object*); @@ -291,7 +282,6 @@ static lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__8___closed LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_buildInductionBody___spec__18(lean_object*); lean_object* l_Lean_Meta_MatcherApp_transform___at_Lean_Meta_MatcherApp_inferMatchType___spec__4(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__3; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_buildInductionBody___spec__43___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__6___boxed(lean_object**); uint8_t l___private_Lean_Util_Trace_0__Lean_checkTraceOption(lean_object*, lean_object*, lean_object*); @@ -301,11 +291,11 @@ LEAN_EXPORT lean_object* l_Lean_Meta_MatcherApp_transform___at_Lean_Tactic_FunIn lean_object* l_Lean_mkApp4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_MatcherApp_inferMatchType___spec__9(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_instInhabitedLevel; -static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__11; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Tactic_FunInd_unpackMutualInduction___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_buildInductionBody___spec__26___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_cleanupAfter_allHeqToEq___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_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at_Lean_Tactic_FunInd_buildInductionBody___spec__12___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*); uint8_t lean_string_dec_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Tactic_FunInd_buildInductionCase___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -314,6 +304,7 @@ LEAN_EXPORT lean_object* l_StateT_pure___at_Lean_Tactic_FunInd_buildInductionBod static lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__7___closed__1; LEAN_EXPORT lean_object* l_Lean_mkFreshFVarId___at_Lean_Tactic_FunInd_buildInductionBody___spec__22___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__3___closed__1; +static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__13; lean_object* l_Lean_throwError___at_Lean_Meta_setInlineAttribute___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__6___closed__2; lean_object* l_Lean_InductiveVal_numTypeFormers(lean_object*); @@ -348,6 +339,7 @@ extern lean_object* l_instInhabitedNat; extern lean_object* l_Lean_Elab_WF_eqnInfoExt; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_buildInductionBody___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_mapTR_loop___at_Lean_mkConstWithLevelParams___spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_index(lean_object*); LEAN_EXPORT lean_object* l_List_filterTR_loop___at_Lean_Tactic_FunInd_deriveUnaryInduction___spec__4___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_buildInductionBody___spec__39___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -357,7 +349,6 @@ extern lean_object* l_instInhabitedPUnit; LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Tactic_FunInd_buildInductionBody___spec__6___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_unpackMutualInduction(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_removeLamda___at_Lean_Tactic_FunInd_buildInductionBody___spec__15___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__15; static lean_object* l_Lean_Elab_Structural_Positions_mapMwith___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__12___closed__4; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_cleanPackedArgs___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__16___lambda__2___closed__1; @@ -371,7 +362,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_MatcherApp_transform___at_Lean_Tactic_FunIn static lean_object* l_Lean_Tactic_FunInd_cleanPackedArgs___lambda__4___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__1(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_withLetDecls_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_Lean_Tactic_FunInd_buildInductionBody___lambda__19___closed__1; static lean_object* l_Lean_Tactic_FunInd_cleanPackedArgs___lambda__5___closed__3; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_cleanupAfter_allHeqToEq___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -380,15 +370,19 @@ lean_object* l_panic___at___private_Lean_Meta_InferType_0__Lean_Meta_checkInferT LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_MatcherApp_Transform_0__Lean_Meta_MatcherApp_forallAltTelescope_x27___at_Lean_Tactic_FunInd_buildInductionBody___spec__42___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_throwError___at_Lean_Elab_Structural_getRecArgInfo___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____closed__1; +size_t lean_ptr_addr(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_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__9; +static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__4; static lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__13___closed__8; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Elab_Structural_eqnInfoExt; -static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__12; size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Tactic_FunInd_foldAndCollect___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_buildInductionBody___spec__17___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__24(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__24(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__2; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_isFunInductName(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Tactic_FunInd_buildInductionBody___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__13___closed__1; @@ -406,11 +400,15 @@ LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_abstractIndependentMVars___lambda_ static lean_object* l_Lean_Tactic_FunInd_cleanPackedArgs___lambda__5___closed__1; lean_object* l_Array_reverse___rarg(lean_object*); uint8_t l_instDecidableNot___rarg(uint8_t); +static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__8; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionCase___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_assertIHs___spec__1___closed__1; LEAN_EXPORT lean_object* l_StateT_lift___at_Lean_Tactic_FunInd_buildInductionBody___spec__1(lean_object*); lean_object* l_Lean_throwError___at_Lean_Expr_abstractRangeM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__7; static lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__4___closed__2; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Array_contains___at_Lean_Meta_setMVarUserNamesAt___spec__1(lean_object*, lean_object*); @@ -427,13 +425,13 @@ static lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__7__ LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_buildInductionBody___spec__16___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_Tactic_FunInd_deriveInductionStructural___spec__7___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__10___closed__4; -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___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_Tactic_FunInd_buildInductionBody___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_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_cleanupAfter_allHeqToEq___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*); uint8_t lean_expr_eqv(lean_object*, lean_object*); +static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_cleanupAfter_allHeqToEq___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Match_Extension_getMatcherInfo_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_buildInductionBody___spec__38___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__2; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_foldAndCollect___spec__22___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_zip___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_buildInductionBody___spec__38___lambda__1(size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -448,26 +446,25 @@ static lean_object* l_Lean_Tactic_FunInd_abstractIndependentMVars___lambda__3___ static lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__2___closed__4; LEAN_EXPORT lean_object* l_Lean_logAt___at_Lean_Tactic_FunInd_buildInductionBody___spec__41___lambda__2___boxed(lean_object*); lean_object* l_Lean_Meta_PProdN_proj(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__17___closed__4; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_foldAndCollect___spec__15___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_log___at_Lean_Tactic_FunInd_buildInductionBody___spec__40___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MVarId_getType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__8___closed__4; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__6(size_t, size_t, lean_object*); static lean_object* l_Lean_Meta_MatcherApp_transform___at_Lean_Tactic_FunInd_buildInductionBody___spec__29___closed__4; static lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__16___closed__1; static lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__14___closed__4; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_foldAndCollect___spec__25(lean_object*); lean_object* l_Lean_Elab_Structural_Positions_numIndices(lean_object*); static lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__8___closed__6; -static lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__19___closed__2; -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___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_Tactic_FunInd_buildInductionBody___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_object*); static lean_object* l_Lean_Tactic_FunInd_buildInductionCase___closed__3; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__8___closed__1; static lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__13___closed__2; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__16___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_registerTraceClass(lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_buildInductionBody___spec__16___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__7___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__15; LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Tactic_FunInd_buildInductionBody___spec__4(lean_object*); lean_object* l_Lean_Meta_kabstract(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkHEqRefl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -484,6 +481,7 @@ lean_object* l_Lean_Name_getPrefix(lean_object*); static lean_object* l_Lean_Tactic_FunInd_cleanPackedArgs___lambda__3___closed__1; LEAN_EXPORT lean_object* l_Nat_foldRevM_loop___at_Lean_Tactic_FunInd_foldAndCollect___spec__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_M_branch___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__27(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_buildInductionBody___spec__35(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_M_tell___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -524,17 +522,17 @@ LEAN_EXPORT lean_object* l_List_filterTR_loop___at_Lean_Tactic_FunInd_deriveIndu LEAN_EXPORT lean_object* l_Lean_PersistentArray_forIn___at_Lean_Tactic_FunInd_cleanupAfter_cleanupAfter_x3f___spec__1(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_buildInductionBody___spec__43___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__8___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__8___closed__2; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__21___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__25___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__25___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Expr_withAppAux___at_Lean_Tactic_FunInd_unpackMutualInduction___spec__1___lambda__3___closed__1; static lean_object* l_Lean_Tactic_FunInd_deriveInduction___lambda__1___closed__1; static lean_object* l_Lean_Tactic_FunInd_deduplicateIHs___closed__1; lean_object* lean_st_ref_get(lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__16___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__17___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_M_exec___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__14___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_withErasedFVars___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__20___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_isFunInductName___lambda__2___closed__2; @@ -543,21 +541,21 @@ LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Tactic_FunInd_foldAndCollec LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Tactic_FunInd_unpackMutualInduction___spec__1___lambda__1___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Tactic_FunInd_foldAndCollect___spec__1___lambda__2___closed__1; lean_object* lean_array_pop(lean_object*); -static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__8; +static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__10; LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Tactic_FunInd_buildInductionBody___spec__4___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__18___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_M_run(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_deriveUnaryInduction___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_buildInductionBody___spec__33___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_buildInductionBody___spec__25___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__8; lean_object* lean_st_mk_ref(lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_withLetDecls___rarg___closed__2; LEAN_EXPORT lean_object* l_Lean_getConstInfoDefn___at_Lean_Tactic_FunInd_deriveUnaryInduction___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_MatcherApp_transform___at_Lean_Tactic_FunInd_buildInductionBody___spec__29___lambda__6___closed__5; LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Tactic_FunInd_buildInductionBody___spec__6___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_to_list(lean_object*); -static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__7; +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___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_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_foldAndCollect___spec__16___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_unpackMutualInduction___lambda__6___closed__11; static lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__10___closed__2; @@ -593,6 +591,7 @@ lean_object* l_Lean_Meta_inferType___boxed(lean_object*, lean_object*, lean_obje static lean_object* l_Lean_logAt___at_Lean_Tactic_FunInd_buildInductionBody___spec__41___lambda__2___closed__4; extern lean_object* l_Lean_levelZero; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__16(lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__17___closed__3; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MVarId_revert(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___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*); @@ -610,7 +609,6 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_deriveIn static lean_object* l_Lean_Tactic_FunInd_removeLamda___rarg___lambda__2___closed__3; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_withLetDecls_go(lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_M_exec(lean_object*); -static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__6; lean_object* l_Lean_Meta_whnfD(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deduplicateIHs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__23___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -624,6 +622,7 @@ lean_object* l_Lean_FVarId_getType(lean_object*, lean_object*, lean_object*, lea LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__24___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_removeLamda___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__16___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__17___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_panic___at_Lean_Expr_appFn_x21___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Tactic_FunInd_foldAndCollect___spec__6___closed__1; lean_object* l_List_lengthTRAux___rarg(lean_object*, lean_object*); @@ -631,16 +630,15 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_abstra LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at_Lean_Tactic_FunInd_foldAndCollect___spec__10___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_cleanupAfter_cleanupAfter_x3f(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__1; -static lean_object* l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__23(lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__9___closed__1; static lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__16___closed__3; lean_object* l_Array_indexOfAux___at_Lean_Meta_getElimExprInfo___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_buildInductionBody___spec__43___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_Lean_Tactic_FunInd_buildInductionBody___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_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___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_EXPORT lean_object* l_Lean_Tactic_FunInd_removeLamda___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__12___closed__2; +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_name_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__5(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -674,7 +672,6 @@ LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__3(lea uint8_t l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_maskArray___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_unpackMutualInduction___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__2; static lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__9___closed__1; static lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__11___closed__1; lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -683,7 +680,9 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_deriveIn LEAN_EXPORT lean_object* l_Lean_Meta_withErasedFVars___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__20(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_PProdN_packLambdas(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkNot(lean_object*); +lean_object* l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_unpackMutualInduction___closed__1; +static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__5; uint8_t l_Lean_LocalDecl_isLet(lean_object*); static lean_object* l_Lean_Expr_withAppAux___at_Lean_Tactic_FunInd_unpackMutualInduction___spec__1___lambda__2___closed__3; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_buildInductionBody___spec__43___lambda__2___closed__2; @@ -701,8 +700,8 @@ static lean_object* l_Lean_Meta_MatcherApp_transform___at_Lean_Tactic_FunInd_bui static lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__7___closed__2; lean_object* l_Lean_Expr_appFn_x21(lean_object*); static lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__8___closed__3; +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_forallBoundedTelescope___at_Lean_Tactic_FunInd_buildInductionBody___spec__14___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Tactic_FunInd_withLetDecls___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_cleanPackedArgs___lambda__5___closed__4; LEAN_EXPORT lean_object* l_StateT_bind___at_Lean_Tactic_FunInd_buildInductionBody___spec__3(lean_object*, lean_object*); @@ -714,19 +713,19 @@ LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__25(lean_o lean_object* l_Lean_Elab_Structural_argsInGroup(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_foldAndCollect___spec__24(lean_object*); static lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__11___closed__2; -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__25(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__25(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__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_EXPORT lean_object* l_Lean_Tactic_FunInd_M_ask___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__17___closed__1; static lean_object* l_Lean_Elab_Structural_Positions_mapMwith___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__12___closed__5; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_cleanupAfter_allHeqToEq___spec__5(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_foldAndCollect___spec__17(lean_object*); -static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__4; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_buildInductionBody___spec__43___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_buildInductionBody___spec__31(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MVarId_assert(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__5___boxed(lean_object**); +static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__5; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deduplicateIHs___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_foldAndCollect___spec__18___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_M_localMapM___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -748,7 +747,8 @@ LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at_Lean_Tactic_FunInd_mkLambda static lean_object* l_Lean_Tactic_FunInd_abstractIndependentMVars___closed__2; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkConstWithLevelParams___at_Lean_Meta_mkSimpCongrTheorem___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__5___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__17___closed__2; +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__20___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_unpackMutualInduction___lambda__6___closed__8; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_buildInductionBody___spec__43(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -758,16 +758,16 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_buildInductio LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__9(lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_throwError___at_Lean_LMVarId_getLevel___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_inheritedTraceOptions; +static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__12; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__16(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__13; lean_object* l_Lean_MessageData_ofExpr(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_buildInductionBody___spec__28___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Tactic_FunInd_buildInductionBody___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__24___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Structural_IndGroupInfo_ofInductiveVal(lean_object*); static lean_object* l_panic___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__13___closed__1; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_buildInductionBody___spec__27___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__11; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__13(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_forallTelescopeReducingAuxAux___rarg(uint8_t, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -796,7 +796,6 @@ static lean_object* l_Lean_Tactic_FunInd_abstractIndependentMVars___closed__4; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_unpackMutualInduction___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_name_append_index_after(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__8___boxed(lean_object**); -static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__14; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionCase___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_foldAndCollect___spec__20___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isFVarOf(lean_object*, lean_object*); @@ -805,6 +804,7 @@ static lean_object* l_Lean_Tactic_FunInd_cleanPackedArgs___lambda__4___closed__1 static lean_object* l_panic___at_Lean_Tactic_FunInd_foldAndCollect___spec__5___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Structural_Positions_groupAndSort___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_MatcherApp_transform___at_Lean_Tactic_FunInd_buildInductionBody___spec__29___lambda__4___boxed(lean_object**); +static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__14; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__15___closed__3; lean_object* l_Lean_Meta_MatcherApp_inferMatchType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -825,6 +825,7 @@ lean_object* l_Lean_instAddErrorMessageContextOfAddMessageContextOfMonad___rarg( lean_object* l_panic___at_Lean_Elab_Structural_Positions_groupAndSort___spec__4(lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInduction(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_heqToEq(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__3; static lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__7___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_M_localMapM___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Name_hasMacroScopes(lean_object*); @@ -841,7 +842,7 @@ static lean_object* l_Lean_Tactic_FunInd_buildInductionCase___closed__1; static lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___closed__2; static lean_object* l_Lean_Tactic_FunInd_cleanupAfter_cleanupAfter_x3f___lambda__1___closed__1; static lean_object* l_Lean_Tactic_FunInd_unpackMutualInduction___lambda__6___closed__10; -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__19___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__19___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_MatcherApp_Transform_0__Lean_Meta_MatcherApp_forallAltTelescope_x27___at_Lean_Tactic_FunInd_buildInductionBody___spec__42(lean_object*); LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Tactic_FunInd_buildInductionCase___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_Tactic_FunInd_cleanPackedArgs___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -855,12 +856,11 @@ LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_M2_branch(lean_object*); static lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__10___closed__6; lean_object* l_Lean_Expr_app___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__7(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_foldAndCollect___spec__24___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_buildInductionBody___spec__20___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_mkLambdaFVarsMasked(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__6; lean_object* l_Lean_Meta_mapErrorImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__6___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__13___closed__2; static lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__13___closed__2; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -871,7 +871,6 @@ LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda static lean_object* l_Lean_Tactic_FunInd_abstractIndependentMVars___lambda__3___closed__1; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_foldAndCollect___spec__15(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__16___lambda__2___closed__4; -static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__8; static lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__11___closed__2; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_projectMutualInduct___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_brecOnSuffix; @@ -887,19 +886,21 @@ lean_object* l_Lean_instantiateMVars___at___private_Lean_Meta_Basic_0__Lean_Meta static lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__16___lambda__4___closed__2; static lean_object* l_panic___at_Lean_Tactic_FunInd_buildInductionBody___spec__10___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_buildInductionBody___spec__38___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__2; lean_object* l_Lean_PersistentHashMap_insert___at_Lean_MVarId_assign___spec__1(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_getLocalInstances(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__10___closed__2; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* l_Lean_observing_x3f___at_Lean_MVarId_iffOfEq___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_cleanupAfter_cleanupAfter_x3f___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__6; static lean_object* l_Lean_getConstInfo___at_Lean_Tactic_FunInd_foldAndCollect___spec__3___closed__1; lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__19(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__19(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__14(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_cleanPackedArgs___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_MVarId_assign___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__11; LEAN_EXPORT lean_object* l_Lean_Meta_MatcherApp_transform___at_Lean_Tactic_FunInd_buildInductionBody___spec__29___lambda__3___boxed(lean_object**); lean_object* l_Lean_Meta_mkEqRefl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_unpackMutualInduction___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -937,9 +938,10 @@ static lean_object* l_Lean_Meta_MatcherApp_transform___at_Lean_Tactic_FunInd_bui LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_maskArray___rarg(lean_object*, lean_object*); lean_object* l_Lean_mkFreshFVarId___at___private_Lean_Meta_Basic_0__Lean_Meta_forallTelescopeReducingAuxAux_process___spec__1___rarg(lean_object*, lean_object*); lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(lean_object*, lean_object*); lean_object* l_Lean_Meta_MatcherApp_toExpr(lean_object*); +static lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__20___closed__1; static lean_object* l_Lean_Elab_Structural_Positions_groupAndSort___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__3___closed__3; -static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__12; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_panic_fn(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_isFunInductName___lambda__1___boxed(lean_object*); @@ -956,14 +958,11 @@ LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__12( lean_object* lean_get_match_equations_for(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Structural_Positions_groupAndSort___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__3___closed__2; -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__5(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_cleanupAfter_cleanupAfter_x3f___spec__4___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_getAppFn(lean_object*); lean_object* l_Lean_Meta_withLCtx___at___private_Lean_Meta_Basic_0__Lean_Meta_mkLevelErrorMessageCore___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_projectMutualInduct___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__15(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__6; static lean_object* l_Lean_Elab_Structural_Positions_mapMwith___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__12___closed__3; static lean_object* l_Lean_Tactic_FunInd_M_branch___rarg___closed__1; static lean_object* l_Lean_Elab_Structural_Positions_groupAndSort___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__3___closed__4; @@ -991,10 +990,8 @@ lean_object* l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_obj lean_object* l_Array_ofSubarray___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_withLetDecls_go___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__19___lambda__3___closed__5; -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470_(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe___at_Lean_Tactic_FunInd_M_localMapM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___closed__2; -static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__9; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__7___boxed(lean_object**); lean_object* l_Array_back___rarg(lean_object*, lean_object*); @@ -1010,7 +1007,6 @@ static lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__15_ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_projectMutualInduct___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__10___closed__2; static lean_object* l_Lean_Meta_MatcherApp_transform___at_Lean_Tactic_FunInd_buildInductionBody___spec__29___lambda__2___closed__2; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_lambdaTelescope___at_Lean_Tactic_FunInd_buildInductionBody___spec__34___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_mk(lean_object*); static lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__16___closed__4; @@ -1031,33 +1027,36 @@ lean_object* l_Lean_Meta_elimOptParam___lambda__1___boxed(lean_object*, lean_obj size_t lean_usize_add(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Tactic_FunInd_foldAndCollect___spec__1(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__5___closed__1; -static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__5; static lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__13___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_buildInductionBody___spec__31___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_forInAux___at_Lean_Tactic_FunInd_cleanupAfter_allHeqToEq___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_buildInductionBody___spec__43___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__4; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_maskArray___rarg___boxed(lean_object*, lean_object*); extern lean_object* l_Lean_instInhabitedName; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_unpackMutualInduction___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Tactic_FunInd_foldAndCollect___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__12; lean_object* lean_array_uget(lean_object*, size_t); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_fvar___override(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_buildInductionBody___spec__24___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___closed__1; size_t lean_array_size(lean_object*); LEAN_EXPORT uint8_t l_Lean_Expr_withAppAux___at_Lean_Tactic_FunInd_unpackMutualInduction___spec__1___lambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__19___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_buildInductionBody___spec__43___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_buildInductionBody___spec__44(lean_object*, size_t, size_t, lean_object*); +static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__7; extern lean_object* l_Lean_instInhabitedDefinitionVal; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__16___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_forInUnsafe_loop___at_Lean_Tactic_FunInd_buildInductionBody___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*); LEAN_EXPORT uint8_t l_Lean_Tactic_FunInd_isFunInductName___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__14(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Loop_forIn_loop___at_Lean_Tactic_FunInd_mkLambdaFVarsMasked___spec__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__23___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_buildInductionBody___spec__26___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_instInhabitedOfMonad___rarg(lean_object*, lean_object*); lean_object* l_Lean_getConstInfoInduct___at_Lean_Meta_mkInjectiveTheorems___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1066,11 +1065,12 @@ lean_object* l_Lean_addTrace___at_Lean_Meta_processPostponed_loop___spec__2(lean lean_object* l___private_Lean_Meta_Match_MatcherApp_Transform_0__Lean_Meta_MatcherApp_withUserNamesImpl___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__16___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__17(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_hasConst___at_Lean_Elab_Structural_getRecArgInfo___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__7; static lean_object* l_Lean_Expr_withAppAux___at_Lean_Tactic_FunInd_unpackMutualInduction___spec__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__7(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_cleanupAfter_cleanupAfter_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_MatcherApp_transform___at_Lean_Tactic_FunInd_buildInductionBody___spec__29___lambda__2___closed__3; +static lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__27___closed__1; +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___closed__1; lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallTelescopeReducingAux___rarg(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__14(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_projectMutualInduct___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1085,6 +1085,7 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_derive static lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__8___closed__1; static lean_object* l_Lean_Tactic_FunInd_cleanPackedArgs___lambda__4___closed__4; LEAN_EXPORT lean_object* l_Lean_PersistentArray_forInAux___at_Lean_Tactic_FunInd_cleanupAfter_allHeqToEq___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__11; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__19___lambda__3___closed__4; lean_object* l_Lean_Meta_Match_MatcherInfo_getNumDiscrEqs(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_buildInductionBody___spec__38___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1106,6 +1107,7 @@ lean_object* l_Lean_Meta_mkFreshExprSyntheticOpaqueMVar(lean_object*, lean_objec LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_foldAndCollect___spec__19___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__2(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__9; lean_object* l_Lean_Expr_headBeta(lean_object*); static lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__4___closed__3; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__18___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1115,15 +1117,14 @@ lean_object* lean_array_get_size(lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__9___boxed(lean_object**); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_buildInductionBody___spec__27___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__8(lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Match_forallAltTelescope___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____closed__1; -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__22___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t l_Lean_Expr_isMData(lean_object*); LEAN_EXPORT lean_object* l_Lean_isTracingEnabledFor___at_Lean_Tactic_FunInd_buildInductionCase___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_buildInductionBody___spec__38___lambda__3(size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_forIn___at_Lean_Tactic_FunInd_cleanupAfter_allHeqToEq___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9___closed__1; lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_forallBoundedTelescope___at_Lean_Tactic_FunInd_buildInductionBody___spec__14___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); @@ -1158,11 +1159,11 @@ LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__2(l LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__20___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_beta(lean_object*, lean_object*); lean_object* l_Lean_mkApp5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__9; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_cleanupAfter_go(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__21(lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Elab_Structural_Positions_mapMwith___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__12___closed__6; static lean_object* l_panic___at_Lean_Tactic_FunInd_buildInductionBody___spec__10___closed__2; +lean_object* l_Lean_Expr_mdataExpr_x21(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_deriveInductionStructural___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_Tactic_FunInd_foldAndCollect___lambda__10___closed__5; static lean_object* l_Lean_Elab_Structural_Positions_mapMwith___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__12___closed__2; @@ -1184,11 +1185,11 @@ lean_object* l_Lean_Expr_mvarId_x21(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__8(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_StateT_lift___at_Lean_Tactic_FunInd_buildInductionBody___spec__2(lean_object*); lean_object* l_Lean_InductiveVal_numCtors(lean_object*); -static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__3; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_foldAndCollect___spec__23___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Split_0__Lean_Meta_Split_generalizeMatchDiscrs___spec__1(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__3___boxed(lean_object**); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__3(lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__3; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_buildInductionBody___spec__25(lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_MatcherApp_transform___at_Lean_Tactic_FunInd_buildInductionBody___spec__29___lambda__6___closed__1; @@ -1204,6 +1205,7 @@ static lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__17___clo LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Tactic_FunInd_buildInductionCase___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_expr_instantiate1(lean_object*, lean_object*); lean_object* l___private_Init_Data_Repr_0__Nat_reprFast(lean_object*); +static lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__27___closed__2; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__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_Lean_Meta_MatcherApp_transform___at_Lean_Tactic_FunInd_buildInductionBody___spec__29___lambda__2___closed__1; lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_instantiateForallAux(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1215,6 +1217,7 @@ LEAN_EXPORT lean_object* l_Lean_isTracingEnabledFor___at_Lean_Tactic_FunInd_buil static lean_object* l_Lean_Elab_Structural_Positions_groupAndSort___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__3___closed__6; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_isFunInductName___lambda__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_lambdaTelescope___at_Lean_Tactic_FunInd_buildInductionBody___spec__34(lean_object*); +static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__4; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__19___lambda__1___boxed(lean_object*, lean_object*); lean_object* l_Lean_Meta_isProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1226,7 +1229,6 @@ static lean_object* l_Lean_Tactic_FunInd_withLetDecls___rarg___closed__1; static lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__3___closed__4; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__5___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__12___closed__2; -static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__1; lean_object* l_Lean_mkFreshFVarId___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_buildInductionBody___closed__2; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -8976,18 +8978,20 @@ LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__24(lean_o _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_inc(x_1); lean_inc(x_6); -x_13 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_foldAndCollect___lambda__6___boxed), 7, 1); +x_13 = lean_alloc_closure((void*)(l_Lean_Meta_mkLetFun), 8, 2); lean_closure_set(x_13, 0, x_6); -x_14 = lean_expr_instantiate1(x_1, x_6); +lean_closure_set(x_13, 1, x_1); +x_14 = lean_expr_instantiate1(x_2, x_6); x_15 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_foldAndCollect), 10, 4); -lean_closure_set(x_15, 0, x_2); -lean_closure_set(x_15, 1, x_3); -lean_closure_set(x_15, 2, x_4); +lean_closure_set(x_15, 0, x_3); +lean_closure_set(x_15, 1, x_4); +lean_closure_set(x_15, 2, x_5); lean_closure_set(x_15, 3, x_14); x_16 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_foldAndCollect___lambda__23), 9, 2); lean_closure_set(x_16, 0, x_6); -lean_closure_set(x_16, 1, x_5); +lean_closure_set(x_16, 1, x_1); x_17 = lean_alloc_closure((void*)(l_StateT_bind___at_Lean_Tactic_FunInd_foldAndCollect___spec__8___rarg), 8, 2); lean_closure_set(x_17, 0, x_15); lean_closure_set(x_17, 1, x_16); @@ -9140,7 +9144,7 @@ lean_inc(x_2); x_76 = l_Lean_Tactic_FunInd_foldAndCollect(x_2, x_3, x_4, x_69, x_75, x_7, x_8, x_9, x_10, x_73); 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; uint8_t x_82; lean_object* x_83; +lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; uint8_t x_82; uint8_t x_83; lean_object* x_84; x_77 = lean_ctor_get(x_76, 0); lean_inc(x_77); x_78 = lean_ctor_get(x_76, 1); @@ -9151,84 +9155,84 @@ lean_inc(x_79); x_80 = lean_ctor_get(x_77, 1); lean_inc(x_80); lean_dec(x_77); -lean_inc(x_79); lean_inc(x_4); lean_inc(x_2); x_81 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_foldAndCollect___lambda__24___boxed), 12, 5); -lean_closure_set(x_81, 0, x_70); -lean_closure_set(x_81, 1, x_2); -lean_closure_set(x_81, 2, x_3); -lean_closure_set(x_81, 3, x_4); -lean_closure_set(x_81, 4, x_79); +lean_closure_set(x_81, 0, x_79); +lean_closure_set(x_81, 1, x_70); +lean_closure_set(x_81, 2, x_2); +lean_closure_set(x_81, 3, x_3); +lean_closure_set(x_81, 4, x_4); x_82 = 0; +x_83 = 0; lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -x_83 = l_Lean_Meta_withLetDecl___at_Lean_Tactic_FunInd_foldAndCollect___spec__10___rarg(x_67, x_74, x_79, x_81, x_82, x_80, x_7, x_8, x_9, x_10, x_78); -if (lean_obj_tag(x_83) == 0) +x_84 = l_Lean_Meta_withLocalDecl___at_Lean_Tactic_FunInd_foldAndCollect___spec__9___rarg(x_67, x_82, x_74, x_81, x_83, x_80, x_7, x_8, x_9, x_10, x_78); +if (lean_obj_tag(x_84) == 0) { -lean_object* x_84; lean_object* x_85; uint8_t x_86; -x_84 = lean_ctor_get(x_83, 0); -lean_inc(x_84); -x_85 = lean_ctor_get(x_83, 1); +lean_object* x_85; lean_object* x_86; uint8_t x_87; +x_85 = lean_ctor_get(x_84, 0); lean_inc(x_85); -lean_dec(x_83); -x_86 = !lean_is_exclusive(x_84); -if (x_86 == 0) +x_86 = lean_ctor_get(x_84, 1); +lean_inc(x_86); +lean_dec(x_84); +x_87 = !lean_is_exclusive(x_85); +if (x_87 == 0) { -x_13 = x_84; -x_14 = x_85; +x_13 = x_85; +x_14 = x_86; goto block_55; } else { -lean_object* x_87; lean_object* x_88; lean_object* x_89; -x_87 = lean_ctor_get(x_84, 0); -x_88 = lean_ctor_get(x_84, 1); +lean_object* x_88; lean_object* x_89; lean_object* x_90; +x_88 = lean_ctor_get(x_85, 0); +x_89 = lean_ctor_get(x_85, 1); +lean_inc(x_89); lean_inc(x_88); -lean_inc(x_87); -lean_dec(x_84); -x_89 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_89, 0, x_87); -lean_ctor_set(x_89, 1, x_88); -x_13 = x_89; -x_14 = x_85; +lean_dec(x_85); +x_90 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_90, 0, x_88); +lean_ctor_set(x_90, 1, x_89); +x_13 = x_90; +x_14 = x_86; goto block_55; } } else { -uint8_t x_90; +uint8_t x_91; lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_4); lean_dec(x_2); -x_90 = !lean_is_exclusive(x_83); -if (x_90 == 0) +x_91 = !lean_is_exclusive(x_84); +if (x_91 == 0) { -return x_83; +return x_84; } else { -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_object* x_92; lean_object* x_93; lean_object* x_94; +x_92 = lean_ctor_get(x_84, 0); +x_93 = lean_ctor_get(x_84, 1); +lean_inc(x_93); 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; +lean_dec(x_84); +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_94; +uint8_t x_95; lean_dec(x_74); lean_dec(x_70); lean_dec(x_67); @@ -9239,29 +9243,29 @@ lean_dec(x_7); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_94 = !lean_is_exclusive(x_76); -if (x_94 == 0) +x_95 = !lean_is_exclusive(x_76); +if (x_95 == 0) { return x_76; } else { -lean_object* x_95; lean_object* x_96; lean_object* x_97; -x_95 = lean_ctor_get(x_76, 0); -x_96 = lean_ctor_get(x_76, 1); +lean_object* x_96; lean_object* x_97; lean_object* x_98; +x_96 = lean_ctor_get(x_76, 0); +x_97 = lean_ctor_get(x_76, 1); +lean_inc(x_97); lean_inc(x_96); -lean_inc(x_95); lean_dec(x_76); -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; +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_98; +uint8_t x_99; lean_dec(x_70); lean_dec(x_69); lean_dec(x_67); @@ -9272,23 +9276,23 @@ lean_dec(x_7); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_98 = !lean_is_exclusive(x_71); -if (x_98 == 0) +x_99 = !lean_is_exclusive(x_71); +if (x_99 == 0) { return x_71; } else { -lean_object* x_99; lean_object* x_100; lean_object* x_101; -x_99 = lean_ctor_get(x_71, 0); -x_100 = lean_ctor_get(x_71, 1); +lean_object* x_100; lean_object* x_101; lean_object* x_102; +x_100 = lean_ctor_get(x_71, 0); +x_101 = lean_ctor_get(x_71, 1); +lean_inc(x_101); lean_inc(x_100); -lean_inc(x_99); lean_dec(x_71); -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; +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; } } } @@ -9938,7 +9942,7 @@ LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__24___boxe { lean_object* x_13; x_13 = l_Lean_Tactic_FunInd_foldAndCollect___lambda__24(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_1); +lean_dec(x_2); return x_13; } } @@ -39765,7 +39769,190 @@ return x_70; } } } -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___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) { +static lean_object* _init_l_Lean_Tactic_FunInd_buildInductionBody___lambda__17___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean.Expr", 9, 9); +return x_1; +} +} +static lean_object* _init_l_Lean_Tactic_FunInd_buildInductionBody___lambda__17___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("_private.Lean.Expr.0.Lean.Expr.updateMData!Impl", 47, 47); +return x_1; +} +} +static lean_object* _init_l_Lean_Tactic_FunInd_buildInductionBody___lambda__17___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mdata expected", 14, 14); +return x_1; +} +} +static lean_object* _init_l_Lean_Tactic_FunInd_buildInductionBody___lambda__17___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_Tactic_FunInd_buildInductionBody___lambda__17___closed__1; +x_2 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__17___closed__2; +x_3 = lean_unsigned_to_nat(1724u); +x_4 = lean_unsigned_to_nat(17u); +x_5 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__17___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_Tactic_FunInd_buildInductionBody___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_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +uint8_t x_15; +x_15 = l_Lean_Expr_isMData(x_6); +if (x_15 == 0) +{ +lean_object* x_16; lean_object* x_17; +x_16 = lean_box(0); +x_17 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__16(x_1, x_2, x_3, x_4, x_5, x_6, x_16, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +return x_17; +} +else +{ +lean_object* x_18; lean_object* x_19; +x_18 = l_Lean_Expr_mdataExpr_x21(x_6); +x_19 = l_Lean_Tactic_FunInd_buildInductionBody(x_4, x_5, x_1, x_2, x_3, 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_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_19, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_19, 1); +lean_inc(x_22); +if (lean_is_exclusive(x_19)) { + lean_ctor_release(x_19, 0); + lean_ctor_release(x_19, 1); + x_23 = x_19; +} else { + lean_dec_ref(x_19); + x_23 = lean_box(0); +} +x_24 = lean_ctor_get(x_20, 1); +lean_inc(x_24); +if (lean_is_exclusive(x_20)) { + lean_ctor_release(x_20, 0); + lean_ctor_release(x_20, 1); + x_25 = x_20; +} else { + lean_dec_ref(x_20); + x_25 = lean_box(0); +} +x_26 = lean_ctor_get(x_21, 0); +lean_inc(x_26); +x_27 = lean_ctor_get(x_21, 1); +lean_inc(x_27); +if (lean_is_exclusive(x_21)) { + lean_ctor_release(x_21, 0); + lean_ctor_release(x_21, 1); + x_28 = x_21; +} else { + lean_dec_ref(x_21); + x_28 = lean_box(0); +} +if (lean_obj_tag(x_6) == 10) +{ +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_6, 0); +lean_inc(x_34); +x_35 = lean_ctor_get(x_6, 1); +lean_inc(x_35); +x_36 = lean_ptr_addr(x_35); +lean_dec(x_35); +x_37 = lean_ptr_addr(x_26); +x_38 = lean_usize_dec_eq(x_36, x_37); +if (x_38 == 0) +{ +lean_object* x_39; +lean_dec(x_6); +x_39 = l_Lean_Expr_mdata___override(x_34, x_26); +x_29 = x_39; +goto block_33; +} +else +{ +lean_dec(x_34); +lean_dec(x_26); +x_29 = x_6; +goto block_33; +} +} +else +{ +lean_object* x_40; lean_object* x_41; +lean_dec(x_26); +lean_dec(x_6); +x_40 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__17___closed__4; +x_41 = l_panic___at_Lean_Expr_appFn_x21___spec__1(x_40); +x_29 = x_41; +goto block_33; +} +block_33: +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; +if (lean_is_scalar(x_28)) { + x_30 = lean_alloc_ctor(0, 2, 0); +} else { + x_30 = x_28; +} +lean_ctor_set(x_30, 0, x_29); +lean_ctor_set(x_30, 1, x_27); +if (lean_is_scalar(x_25)) { + x_31 = lean_alloc_ctor(0, 2, 0); +} else { + x_31 = x_25; +} +lean_ctor_set(x_31, 0, x_30); +lean_ctor_set(x_31, 1, x_24); +if (lean_is_scalar(x_23)) { + x_32 = lean_alloc_ctor(0, 2, 0); +} else { + x_32 = x_23; +} +lean_ctor_set(x_32, 0, x_31); +lean_ctor_set(x_32, 1, x_22); +return x_32; +} +} +else +{ +uint8_t x_42; +lean_dec(x_6); +x_42 = !lean_is_exclusive(x_19); +if (x_42 == 0) +{ +return x_19; +} +else +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_19, 0); +x_44 = lean_ctor_get(x_19, 1); +lean_inc(x_44); +lean_inc(x_43); +lean_dec(x_19); +x_45 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_45, 0, x_43); +lean_ctor_set(x_45, 1, x_44); +return x_45; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___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, 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; @@ -39869,7 +40056,7 @@ return x_33; } } } -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___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, 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_Tactic_FunInd_buildInductionBody___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) { _start: { lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; @@ -39887,7 +40074,7 @@ lean_ctor_set(x_16, 1, x_11); return x_16; } } -static lean_object* _init_l_Lean_Tactic_FunInd_buildInductionBody___lambda__19___closed__1() { +static lean_object* _init_l_Lean_Tactic_FunInd_buildInductionBody___lambda__20___closed__1() { _start: { lean_object* x_1; @@ -39895,12 +40082,12 @@ x_1 = lean_mk_string_unchecked("Lean.Tactic.FunInd.buildInductionBody", 37, 37); return x_1; } } -static lean_object* _init_l_Lean_Tactic_FunInd_buildInductionBody___lambda__19___closed__2() { +static lean_object* _init_l_Lean_Tactic_FunInd_buildInductionBody___lambda__20___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_Tactic_FunInd_foldAndCollect___lambda__8___closed__1; -x_2 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__19___closed__1; +x_2 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__20___closed__1; x_3 = lean_unsigned_to_nat(581u); x_4 = lean_unsigned_to_nat(40u); x_5 = l_List_forIn_loop___at_Lean_Tactic_FunInd_foldAndCollect___spec__6___closed__3; @@ -39908,7 +40095,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_Tactic_FunInd_buildInductionBody___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_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___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_object* x_12, lean_object* x_13) { _start: { lean_object* x_14; lean_object* x_15; uint8_t x_16; @@ -39924,7 +40111,7 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_17 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__19___closed__2; +x_17 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__20___closed__2; x_18 = l_panic___at_Lean_Tactic_FunInd_buildInductionBody___spec__13(x_17, x_7, x_8, x_9, x_10, x_11, x_12, x_13); return x_18; } @@ -40233,11 +40420,11 @@ return x_91; } } } -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___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_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___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_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; uint8_t x_15; lean_object* x_16; -x_13 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_buildInductionBody___lambda__19___boxed), 13, 4); +x_13 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_buildInductionBody___lambda__20___boxed), 13, 4); lean_closure_set(x_13, 0, x_1); lean_closure_set(x_13, 1, x_4); lean_closure_set(x_13, 2, x_2); @@ -40248,11 +40435,11 @@ x_16 = l_Lean_Meta_forallBoundedTelescope___at_Lean_Tactic_FunInd_buildInduction return x_16; } } -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___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_Tactic_FunInd_buildInductionBody___lambda__22(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_12 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_buildInductionBody___lambda__20), 12, 3); +x_12 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_buildInductionBody___lambda__21), 12, 3); lean_closure_set(x_12, 0, x_1); lean_closure_set(x_12, 1, x_2); lean_closure_set(x_12, 2, x_3); @@ -40263,7 +40450,7 @@ x_14 = l_Lean_Tactic_FunInd_M2_branch___rarg(x_13, x_5, x_6, x_7, x_8, x_9, x_10 return x_14; } } -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__22(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__23(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; @@ -40285,7 +40472,7 @@ lean_ctor_set(x_16, 1, x_9); return x_16; } } -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__23(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_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_Tactic_FunInd_buildInductionBody___lambda__24(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_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; @@ -40300,7 +40487,7 @@ x_15 = l_Lean_Tactic_FunInd_M2_branch___rarg(x_14, x_7, x_8, x_9, x_10, x_11, x_ return x_15; } } -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__24(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_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_Tactic_FunInd_buildInductionBody___lambda__25(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { lean_object* x_17; uint8_t x_18; @@ -40347,14 +40534,14 @@ lean_dec(x_22); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_26 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_buildInductionBody___lambda__17), 11, 3); +x_26 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_buildInductionBody___lambda__18), 11, 3); lean_closure_set(x_26, 0, x_5); lean_closure_set(x_26, 1, x_6); lean_closure_set(x_26, 2, x_7); -x_27 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_buildInductionBody___lambda__18___boxed), 11, 2); +x_27 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_buildInductionBody___lambda__19___boxed), 11, 2); lean_closure_set(x_27, 0, x_24); lean_closure_set(x_27, 1, x_25); -x_28 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_buildInductionBody___lambda__23), 13, 4); +x_28 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_buildInductionBody___lambda__24), 13, 4); lean_closure_set(x_28, 0, x_8); lean_closure_set(x_28, 1, x_5); lean_closure_set(x_28, 2, x_6); @@ -40547,7 +40734,7 @@ return x_69; } } } -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__25(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_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_Tactic_FunInd_buildInductionBody___lambda__26(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { uint8_t x_15; lean_object* x_16; @@ -40580,7 +40767,7 @@ x_22 = lean_ctor_get(x_18, 1); lean_inc(x_22); lean_dec(x_18); x_23 = lean_box(0); -x_24 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__16(x_2, x_3, x_4, x_5, x_6, x_1, x_23, x_22, x_21, x_10, x_11, x_12, x_13, x_20); +x_24 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__17(x_2, x_3, x_4, x_5, x_6, x_1, x_23, x_22, x_21, x_10, x_11, x_12, x_13, x_20); return x_24; } else @@ -40603,7 +40790,7 @@ lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); -x_29 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_buildInductionBody___lambda__16___boxed), 14, 6); +x_29 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_buildInductionBody___lambda__17___boxed), 14, 6); lean_closure_set(x_29, 0, x_2); lean_closure_set(x_29, 1, x_3); lean_closure_set(x_29, 2, x_4); @@ -40662,7 +40849,7 @@ lean_dec(x_83); lean_dec(x_41); lean_dec(x_40); x_87 = lean_box(0); -x_88 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__24(x_28, x_29, x_36, x_6, x_2, x_3, x_4, x_5, x_87, x_27, x_26, x_10, x_11, x_12, x_13, x_39); +x_88 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__25(x_28, x_29, x_36, x_6, x_2, x_3, x_4, x_5, x_87, x_27, x_26, x_10, x_11, x_12, x_13, x_39); return x_88; } else @@ -40685,7 +40872,7 @@ lean_object* x_94; lean_object* x_95; lean_dec(x_41); lean_dec(x_40); x_94 = lean_box(0); -x_95 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__24(x_28, x_29, x_36, x_6, x_2, x_3, x_4, x_5, x_94, x_27, x_26, x_10, x_11, x_12, x_13, x_39); +x_95 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__25(x_28, x_29, x_36, x_6, x_2, x_3, x_4, x_5, x_94, x_27, x_26, x_10, x_11, x_12, x_13, x_39); return x_95; } else @@ -40712,7 +40899,7 @@ lean_object* x_99; lean_object* x_100; lean_dec(x_41); lean_dec(x_40); x_99 = lean_box(0); -x_100 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__24(x_28, x_29, x_36, x_6, x_2, x_3, x_4, x_5, x_99, x_27, x_26, x_10, x_11, x_12, x_13, x_39); +x_100 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__25(x_28, x_29, x_36, x_6, x_2, x_3, x_4, x_5, x_99, x_27, x_26, x_10, x_11, x_12, x_13, x_39); return x_100; } else @@ -40733,17 +40920,17 @@ lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean lean_dec(x_42); lean_inc(x_4); lean_inc(x_3); -x_43 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_buildInductionBody___lambda__17), 11, 3); +x_43 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_buildInductionBody___lambda__18), 11, 3); lean_closure_set(x_43, 0, x_2); lean_closure_set(x_43, 1, x_3); lean_closure_set(x_43, 2, x_4); -x_44 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_buildInductionBody___lambda__18___boxed), 11, 2); +x_44 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_buildInductionBody___lambda__19___boxed), 11, 2); lean_closure_set(x_44, 0, x_40); lean_closure_set(x_44, 1, x_41); -x_45 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_buildInductionBody___lambda__21), 11, 2); +x_45 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_buildInductionBody___lambda__22), 11, 2); lean_closure_set(x_45, 0, x_5); lean_closure_set(x_45, 1, x_4); -x_46 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_buildInductionBody___lambda__22___boxed), 9, 1); +x_46 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_buildInductionBody___lambda__23___boxed), 9, 1); lean_closure_set(x_46, 0, x_3); x_47 = l_Lean_Meta_MatcherApp_transform___at_Lean_Tactic_FunInd_buildInductionBody___spec__29(x_28, x_15, x_15, x_43, x_44, x_45, x_46, x_27, x_26, x_10, x_11, x_12, x_13, x_39); if (lean_obj_tag(x_47) == 0) @@ -41004,7 +41191,7 @@ return x_113; } } } -static lean_object* _init_l_Lean_Tactic_FunInd_buildInductionBody___lambda__26___closed__1() { +static lean_object* _init_l_Lean_Tactic_FunInd_buildInductionBody___lambda__27___closed__1() { _start: { lean_object* x_1; @@ -41012,7 +41199,7 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_buildInductionBody___lambd return x_1; } } -static lean_object* _init_l_Lean_Tactic_FunInd_buildInductionBody___lambda__26___closed__2() { +static lean_object* _init_l_Lean_Tactic_FunInd_buildInductionBody___lambda__27___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -41022,7 +41209,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__26(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_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_Tactic_FunInd_buildInductionBody___lambda__27(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_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; uint8_t x_21; @@ -41033,7 +41220,7 @@ lean_inc(x_16); x_17 = lean_ctor_get(x_15, 1); lean_inc(x_17); lean_dec(x_15); -x_18 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__26___closed__1; +x_18 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__27___closed__1; x_19 = l_Lean_Expr_cleanupAnnotations(x_16); x_20 = l_Lean_Tactic_FunInd_foldAndCollect___lambda__12___closed__2; x_21 = l_Lean_Expr_isConstOf(x_19, x_20); @@ -41046,7 +41233,7 @@ if (x_22 == 0) lean_object* x_23; lean_object* x_24; lean_dec(x_19); x_23 = lean_box(0); -x_24 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__25(x_2, x_4, x_5, x_6, x_3, x_1, x_23, x_8, x_9, x_10, x_11, x_12, x_13, x_17); +x_24 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__26(x_2, x_4, x_5, x_6, x_3, x_1, x_23, x_8, x_9, x_10, x_11, x_12, x_13, x_17); return x_24; } else @@ -41061,7 +41248,7 @@ lean_object* x_28; lean_object* x_29; lean_dec(x_26); lean_dec(x_25); x_28 = lean_box(0); -x_29 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__25(x_2, x_4, x_5, x_6, x_3, x_1, x_28, x_8, x_9, x_10, x_11, x_12, x_13, x_17); +x_29 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__26(x_2, x_4, x_5, x_6, x_3, x_1, x_28, x_8, x_9, x_10, x_11, x_12, x_13, x_17); return x_29; } else @@ -41069,7 +41256,7 @@ else lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; x_30 = l_Lean_Expr_appArg(x_26, lean_box(0)); x_31 = l_Lean_Expr_appFnCleanup(x_26, lean_box(0)); -x_32 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__26___closed__2; +x_32 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__27___closed__2; x_33 = l_Lean_Expr_isConstOf(x_31, x_32); lean_dec(x_31); if (x_33 == 0) @@ -41078,7 +41265,7 @@ lean_object* x_34; lean_object* x_35; lean_dec(x_30); lean_dec(x_25); x_34 = lean_box(0); -x_35 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__25(x_2, x_4, x_5, x_6, x_3, x_1, x_34, x_8, x_9, x_10, x_11, x_12, x_13, x_17); +x_35 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__26(x_2, x_4, x_5, x_6, x_3, x_1, x_34, x_8, x_9, x_10, x_11, x_12, x_13, x_17); return x_35; } else @@ -41143,7 +41330,7 @@ if (x_18 == 0) lean_object* x_19; lean_object* x_20; lean_dec(x_17); x_19 = lean_box(0); -x_20 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__26(x_2, x_6, x_1, x_3, x_4, x_5, x_19, x_7, x_8, x_9, x_10, x_11, x_12, x_16); +x_20 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__27(x_2, x_6, x_1, x_3, x_4, x_5, x_19, x_7, x_8, x_9, x_10, x_11, x_12, x_16); return x_20; } else @@ -41158,7 +41345,7 @@ lean_object* x_24; lean_object* x_25; lean_dec(x_22); lean_dec(x_21); x_24 = lean_box(0); -x_25 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__26(x_2, x_6, x_1, x_3, x_4, x_5, x_24, x_7, x_8, x_9, x_10, x_11, x_12, x_16); +x_25 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__27(x_2, x_6, x_1, x_3, x_4, x_5, x_24, x_7, x_8, x_9, x_10, x_11, x_12, x_16); return x_25; } else @@ -41174,7 +41361,7 @@ lean_dec(x_27); lean_dec(x_26); lean_dec(x_21); x_29 = lean_box(0); -x_30 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__26(x_2, x_6, x_1, x_3, x_4, x_5, x_29, x_7, x_8, x_9, x_10, x_11, x_12, x_16); +x_30 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__27(x_2, x_6, x_1, x_3, x_4, x_5, x_29, x_7, x_8, x_9, x_10, x_11, x_12, x_16); return x_30; } else @@ -41191,7 +41378,7 @@ lean_dec(x_31); lean_dec(x_26); lean_dec(x_21); x_34 = lean_box(0); -x_35 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__26(x_2, x_6, x_1, x_3, x_4, x_5, x_34, x_7, x_8, x_9, x_10, x_11, x_12, x_16); +x_35 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__27(x_2, x_6, x_1, x_3, x_4, x_5, x_34, x_7, x_8, x_9, x_10, x_11, x_12, x_16); return x_35; } else @@ -41209,7 +41396,7 @@ lean_dec(x_31); lean_dec(x_26); lean_dec(x_21); x_39 = lean_box(0); -x_40 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__26(x_2, x_6, x_1, x_3, x_4, x_5, x_39, x_7, x_8, x_9, x_10, x_11, x_12, x_16); +x_40 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__27(x_2, x_6, x_1, x_3, x_4, x_5, x_39, x_7, x_8, x_9, x_10, x_11, x_12, x_16); return x_40; } else @@ -41234,7 +41421,7 @@ lean_dec(x_31); lean_dec(x_26); lean_dec(x_21); x_47 = lean_box(0); -x_48 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__26(x_2, x_6, x_1, x_3, x_4, x_5, x_47, x_7, x_8, x_9, x_10, x_11, x_12, x_16); +x_48 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__27(x_2, x_6, x_1, x_3, x_4, x_5, x_47, x_7, x_8, x_9, x_10, x_11, x_12, x_16); return x_48; } else @@ -42280,11 +42467,20 @@ lean_dec(x_7); return x_15; } } -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__18___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__17___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; +x_15 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__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); +lean_dec(x_7); +return x_15; +} +} +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__19___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { lean_object* x_12; -x_12 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__18(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_12 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__19(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); @@ -42294,20 +42490,20 @@ lean_dec(x_1); return x_12; } } -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__19___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__20___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { lean_object* x_14; -x_14 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__19(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +x_14 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__20(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); lean_dec(x_5); return x_14; } } -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__22___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__23___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { lean_object* x_10; -x_10 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__22(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_10 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__23(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); @@ -42316,29 +42512,29 @@ lean_dec(x_2); return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__24___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__25___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { lean_object* x_17; -x_17 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__24(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_17 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__25(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_9); return x_17; } } -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__25___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__26___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { lean_object* x_15; -x_15 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__25(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +x_15 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__26(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_7); return x_15; } } -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__26___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__27___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { lean_object* x_15; -x_15 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__26(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +x_15 = l_Lean_Tactic_FunInd_buildInductionBody___lambda__27(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_7); return x_15; } @@ -42536,7 +42732,7 @@ return x_33; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; @@ -42544,7 +42740,7 @@ x_8 = l_Lean_MVarId_getType(x_1, x_3, x_4, x_5, x_6, x_7); return x_8; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___closed__1() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___closed__1() { _start: { lean_object* x_1; @@ -42552,7 +42748,7 @@ x_1 = lean_mk_string_unchecked("case", 4, 4); return x_1; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; uint8_t x_8; @@ -42569,14 +42765,14 @@ x_12 = lean_nat_add(x_4, x_9); lean_dec(x_4); lean_inc(x_12); x_13 = l___private_Init_Data_Repr_0__Nat_reprFast(x_12); -x_14 = l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___closed__1; +x_14 = l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___closed__1; x_15 = lean_string_append(x_14, x_13); lean_dec(x_13); x_16 = l_Lean_Tactic_FunInd_removeLamda___rarg___lambda__2___closed__3; x_17 = lean_string_append(x_15, x_16); x_18 = lean_box(0); x_19 = l_Lean_Name_str___override(x_18, x_17); -x_20 = lean_alloc_closure((void*)(l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___lambda__1___boxed), 7, 1); +x_20 = lean_alloc_closure((void*)(l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___lambda__1___boxed), 7, 1); lean_closure_set(x_20, 0, x_11); x_21 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_21, 0, x_19); @@ -42881,208 +43077,6 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__6(size_t x_1, size_t x_2, lean_object* x_3) { -_start: -{ -uint8_t x_4; -x_4 = lean_usize_dec_lt(x_2, x_1); -if (x_4 == 0) -{ -return x_3; -} -else -{ -lean_object* x_5; lean_object* x_6; lean_object* x_7; size_t x_8; size_t x_9; uint8_t x_10; -x_5 = lean_array_uget(x_3, x_2); -x_6 = lean_unsigned_to_nat(0u); -x_7 = lean_array_uset(x_3, x_2, x_6); -x_8 = 1; -x_9 = lean_usize_add(x_2, x_8); -x_10 = !lean_is_exclusive(x_5); -if (x_10 == 0) -{ -lean_object* x_11; uint8_t x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_11 = lean_ctor_get(x_5, 0); -x_12 = 0; -x_13 = lean_box(x_12); -lean_ctor_set(x_5, 0, x_13); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_11); -lean_ctor_set(x_14, 1, x_5); -x_15 = lean_array_uset(x_7, x_2, x_14); -x_2 = x_9; -x_3 = x_15; -goto _start; -} -else -{ -lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_17 = lean_ctor_get(x_5, 0); -x_18 = lean_ctor_get(x_5, 1); -lean_inc(x_18); -lean_inc(x_17); -lean_dec(x_5); -x_19 = 0; -x_20 = lean_box(x_19); -x_21 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_21, 0, x_20); -lean_ctor_set(x_21, 1, x_18); -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_17); -lean_ctor_set(x_22, 1, x_21); -x_23 = lean_array_uset(x_7, x_2, x_22); -x_2 = x_9; -x_3 = x_23; -goto _start; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__8___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; lean_object* x_12; -x_11 = lean_array_push(x_1, x_5); -x_12 = l_Lean_Meta_withLocalDecls_loop___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__8___rarg(x_2, x_3, x_4, x_11, x_6, x_7, x_8, x_9, x_10); -return x_12; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__8___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_10 = lean_array_get_size(x_4); -x_11 = lean_array_get_size(x_1); -x_12 = lean_nat_dec_lt(x_10, x_11); -lean_dec(x_11); -if (x_12 == 0) -{ -lean_object* x_13; -lean_dec(x_10); -lean_dec(x_3); -lean_dec(x_1); -x_13 = lean_apply_6(x_2, x_4, x_5, x_6, x_7, x_8, x_9); -return x_13; -} -else -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_14 = lean_array_fget(x_1, x_10); -lean_dec(x_10); -x_15 = lean_ctor_get(x_14, 1); -lean_inc(x_15); -x_16 = lean_ctor_get(x_14, 0); -lean_inc(x_16); -lean_dec(x_14); -x_17 = lean_ctor_get(x_15, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_15, 1); -lean_inc(x_18); -lean_dec(x_15); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -x_19 = lean_apply_6(x_18, x_4, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_19) == 0) -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; uint8_t x_24; lean_object* x_25; -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_19, 1); -lean_inc(x_21); -lean_dec(x_19); -x_22 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecls_loop___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__8___rarg___lambda__1), 10, 4); -lean_closure_set(x_22, 0, x_4); -lean_closure_set(x_22, 1, x_1); -lean_closure_set(x_22, 2, x_2); -lean_closure_set(x_22, 3, x_3); -x_23 = 0; -x_24 = lean_unbox(x_17); -lean_dec(x_17); -x_25 = l_Lean_Meta_withLocalDecl___at_Lean_Meta_forallTelescopeCompatibleAux___spec__15___rarg(x_16, x_24, x_20, x_22, x_23, x_5, x_6, x_7, x_8, x_21); -return x_25; -} -else -{ -uint8_t x_26; -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_26 = !lean_is_exclusive(x_19); -if (x_26 == 0) -{ -return x_19; -} -else -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_19, 0); -x_28 = lean_ctor_get(x_19, 1); -lean_inc(x_28); -lean_inc(x_27); -lean_dec(x_19); -x_29 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_29, 0, x_27); -lean_ctor_set(x_29, 1, x_28); -return x_29; -} -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__8(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecls_loop___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__8___rarg), 9, 0); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__7___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; lean_object* x_10; -x_9 = l_Lean_Tactic_FunInd_M_run___rarg___closed__1; -x_10 = l_Lean_Meta_withLocalDecls_loop___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__8___rarg(x_2, x_3, x_1, x_9, x_4, x_5, x_6, x_7, x_8); -return x_10; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__7(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecls___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__7___rarg), 8, 0); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__5___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -size_t x_9; size_t x_10; lean_object* x_11; lean_object* x_12; -x_9 = lean_array_size(x_2); -x_10 = 0; -x_11 = l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__6(x_9, x_10, x_2); -x_12 = l_Lean_Meta_withLocalDecls___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__7___rarg(x_1, x_11, x_3, x_4, x_5, x_6, x_7, x_8); -return x_12; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__5(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDeclsD___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__5___rarg), 8, 0); -return x_2; -} -} LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_abstractIndependentMVars___lambda__1(lean_object* x_1, size_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { @@ -43116,14 +43110,14 @@ lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean x_10 = lean_array_get_size(x_1); x_11 = lean_mk_empty_array_with_capacity(x_10); x_12 = lean_unsigned_to_nat(0u); -x_13 = l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2(x_1, x_1, x_10, x_12, lean_box(0), x_11); +x_13 = l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2(x_1, x_1, x_10, x_12, lean_box(0), x_11); x_14 = lean_box_usize(x_2); x_15 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_abstractIndependentMVars___lambda__1___boxed), 9, 3); lean_closure_set(x_15, 0, x_1); lean_closure_set(x_15, 1, x_14); lean_closure_set(x_15, 2, x_3); x_16 = l_Lean_instInhabitedExpr; -x_17 = l_Lean_Meta_withLocalDeclsD___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__5___rarg(x_16, x_13, x_15, x_5, x_6, x_7, x_8, x_9); +x_17 = l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__2___rarg(x_16, x_13, x_15, x_5, x_6, x_7, x_8, x_9); return x_17; } } @@ -43438,11 +43432,11 @@ x_12 = l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_abstractIndependentMVars__ return x_12; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; -x_8 = l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); @@ -43451,11 +43445,11 @@ lean_dec(x_2); return x_8; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; -x_7 = l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_2); lean_dec(x_1); return x_7; @@ -43490,18 +43484,6 @@ lean_dec(x_1); return x_12; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -size_t x_4; size_t x_5; lean_object* x_6; -x_4 = lean_unbox_usize(x_1); -lean_dec(x_1); -x_5 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_6 = l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__6(x_4, x_5, x_3); -return x_6; -} -} LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_abstractIndependentMVars___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { @@ -43861,7 +43843,7 @@ if (x_5 == 0) lean_object* x_6; lean_object* x_7; uint8_t x_8; x_6 = lean_ctor_get(x_2, 0); x_7 = lean_ctor_get(x_2, 1); -x_8 = l_Array_contains___at_Lean_findField_x3f___spec__1(x_1, x_6); +x_8 = l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(x_1, x_6); if (x_8 == 0) { lean_free_object(x_2); @@ -43889,7 +43871,7 @@ x_12 = lean_ctor_get(x_2, 1); lean_inc(x_12); lean_inc(x_11); lean_dec(x_2); -x_13 = l_Array_contains___at_Lean_findField_x3f___spec__1(x_1, x_11); +x_13 = l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(x_1, x_11); if (x_13 == 0) { lean_dec(x_11); @@ -48244,7 +48226,7 @@ static lean_object* _init_l_Lean_Tactic_FunInd_cleanPackedArgs___lambda__5___clo lean_object* x_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_Tactic_FunInd_foldAndCollect___lambda__8___closed__1; x_2 = l_Lean_Tactic_FunInd_cleanPackedArgs___lambda__5___closed__4; -x_3 = lean_unsigned_to_nat(783u); +x_3 = lean_unsigned_to_nat(788u); x_4 = lean_unsigned_to_nat(50u); x_5 = l_List_forIn_loop___at_Lean_Tactic_FunInd_foldAndCollect___spec__6___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -51565,7 +51547,7 @@ static lean_object* _init_l_Lean_Tactic_FunInd_withLetDecls___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_Tactic_FunInd_foldAndCollect___lambda__8___closed__1; x_2 = l_Lean_Tactic_FunInd_withLetDecls___rarg___closed__3; -x_3 = lean_unsigned_to_nat(877u); +x_3 = lean_unsigned_to_nat(882u); x_4 = lean_unsigned_to_nat(2u); x_5 = l_Lean_Tactic_FunInd_withLetDecls___rarg___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -52927,7 +52909,7 @@ return x_35; } } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9___closed__1() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9___closed__1() { _start: { lean_object* x_1; @@ -52935,7 +52917,7 @@ x_1 = lean_mk_string_unchecked("motive_", 7, 7); return x_1; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; uint8_t x_14; @@ -52960,7 +52942,7 @@ x_21 = lean_nat_add(x_5, x_15); lean_dec(x_5); lean_inc(x_21); x_22 = l___private_Init_Data_Repr_0__Nat_reprFast(x_21); -x_23 = l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9___closed__1; +x_23 = l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9___closed__1; x_24 = lean_string_append(x_23, x_22); lean_dec(x_22); x_25 = l_Lean_Tactic_FunInd_removeLamda___rarg___lambda__2___closed__3; @@ -57059,7 +57041,7 @@ static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriv lean_object* x_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_Tactic_FunInd_foldAndCollect___lambda__8___closed__1; x_2 = l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__19___lambda__3___closed__1; -x_3 = lean_unsigned_to_nat(1038u); +x_3 = lean_unsigned_to_nat(1043u); x_4 = lean_unsigned_to_nat(73u); x_5 = l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__19___lambda__3___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -57072,7 +57054,7 @@ static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriv lean_object* x_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_Tactic_FunInd_foldAndCollect___lambda__8___closed__1; x_2 = l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__19___lambda__3___closed__1; -x_3 = lean_unsigned_to_nat(1040u); +x_3 = lean_unsigned_to_nat(1045u); x_4 = lean_unsigned_to_nat(62u); x_5 = l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__19___lambda__3___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -57102,7 +57084,7 @@ static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriv lean_object* x_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_Tactic_FunInd_foldAndCollect___lambda__8___closed__1; x_2 = l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__19___lambda__3___closed__1; -x_3 = lean_unsigned_to_nat(1039u); +x_3 = lean_unsigned_to_nat(1044u); x_4 = lean_unsigned_to_nat(67u); x_5 = l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__19___lambda__3___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -59559,7 +59541,7 @@ if (x_5 == 0) lean_object* x_6; lean_object* x_7; uint8_t x_8; x_6 = lean_ctor_get(x_2, 0); x_7 = lean_ctor_get(x_2, 1); -x_8 = l_Array_contains___at_Lean_findField_x3f___spec__1(x_1, x_6); +x_8 = l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(x_1, x_6); if (x_8 == 0) { lean_free_object(x_2); @@ -59587,7 +59569,7 @@ x_12 = lean_ctor_get(x_2, 1); lean_inc(x_12); lean_inc(x_11); lean_dec(x_2); -x_13 = l_Array_contains___at_Lean_findField_x3f___spec__1(x_1, x_11); +x_13 = l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(x_1, x_11); if (x_13 == 0) { lean_dec(x_11); @@ -60948,7 +60930,7 @@ lean_dec(x_25); x_28 = lean_array_get_size(x_23); x_29 = lean_mk_empty_array_with_capacity(x_28); x_30 = lean_unsigned_to_nat(0u); -x_31 = l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9(x_5, x_23, x_23, x_28, x_30, lean_box(0), x_29, x_17, x_18, x_19, x_20, x_27); +x_31 = l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9(x_5, x_23, x_23, x_28, x_30, lean_box(0), x_29, x_17, x_18, x_19, x_20, x_27); lean_dec(x_23); x_32 = lean_ctor_get(x_31, 0); lean_inc(x_32); @@ -60976,7 +60958,7 @@ lean_closure_set(x_36, 14, x_26); lean_closure_set(x_36, 15, x_15); lean_closure_set(x_36, 16, x_16); x_37 = l_Lean_instInhabitedExpr; -x_38 = l_Lean_Meta_withLocalDeclsD___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__5___rarg(x_37, x_32, x_36, x_17, x_18, x_19, x_20, x_33); +x_38 = l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__2___rarg(x_37, x_32, x_36, x_17, x_18, x_19, x_20, x_33); return x_38; } else @@ -61087,7 +61069,7 @@ static lean_object* _init_l_Lean_Tactic_FunInd_deriveInductionStructural___lambd lean_object* x_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_Tactic_FunInd_foldAndCollect___lambda__8___closed__1; x_2 = l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__19___lambda__3___closed__1; -x_3 = lean_unsigned_to_nat(961u); +x_3 = lean_unsigned_to_nat(966u); x_4 = lean_unsigned_to_nat(6u); x_5 = l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__9___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -61949,7 +61931,7 @@ static lean_object* _init_l_Lean_Tactic_FunInd_deriveInductionStructural___lambd lean_object* x_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_Tactic_FunInd_foldAndCollect___lambda__8___closed__1; x_2 = l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__19___lambda__3___closed__1; -x_3 = lean_unsigned_to_nat(914u); +x_3 = lean_unsigned_to_nat(919u); x_4 = lean_unsigned_to_nat(41u); x_5 = l_List_forIn_loop___at_Lean_Tactic_FunInd_foldAndCollect___spec__6___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -63513,11 +63495,11 @@ lean_dec(x_1); return x_12; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; -x_13 = l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_13 = l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -65073,7 +65055,7 @@ lean_dec(x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { uint8_t x_5; lean_object* x_6; lean_object* x_7; @@ -65085,15 +65067,15 @@ lean_ctor_set(x_7, 1, x_4); return x_7; } } -static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__1() { +static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__1___boxed), 4, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__1___boxed), 4, 0); return x_1; } } -static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__2() { +static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__2() { _start: { uint8_t x_1; uint8_t x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; @@ -65118,7 +65100,7 @@ lean_ctor_set_uint8(x_5, 12, x_2); return x_5; } } -static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__3() { +static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__3() { _start: { lean_object* x_1; @@ -65126,17 +65108,17 @@ x_1 = l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_box(0), lean_box(0)); return x_1; } } -static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__4() { +static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__3; +x_1 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__3; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__5() { +static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__5() { _start: { lean_object* x_1; lean_object* x_2; @@ -65145,23 +65127,23 @@ x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__6() { +static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__6() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__5; +x_1 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__5; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__7() { +static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__7() { _start: { size_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = 5; -x_2 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__6; -x_3 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__5; +x_2 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__6; +x_3 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__5; x_4 = lean_unsigned_to_nat(0u); x_5 = lean_alloc_ctor(0, 4, sizeof(size_t)*1); lean_ctor_set(x_5, 0, x_2); @@ -65172,25 +65154,25 @@ lean_ctor_set_usize(x_5, 4, x_1); return x_5; } } -static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__8() { +static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__4; -x_2 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__7; +x_1 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__4; +x_2 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__7; x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__9() { +static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; uint8_t x_6; lean_object* x_7; x_1 = lean_box(0); -x_2 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__2; -x_3 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__8; +x_2 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__2; +x_3 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__8; x_4 = l_Lean_Tactic_FunInd_M_run___rarg___closed__1; x_5 = lean_unsigned_to_nat(0u); x_6 = 0; @@ -65206,12 +65188,12 @@ lean_ctor_set_uint8(x_7, sizeof(void*)*6 + 1, x_6); return x_7; } } -static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__10() { +static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_unsigned_to_nat(0u); -x_2 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__4; +x_2 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__4; x_3 = lean_alloc_ctor(0, 9, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_1); @@ -65225,22 +65207,22 @@ lean_ctor_set(x_3, 8, x_2); return x_3; } } -static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__11() { +static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__11() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__4; +x_1 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__4; x_2 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_2, 0, x_1); lean_ctor_set(x_2, 1, x_1); return x_2; } } -static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__12() { +static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__12() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__4; +x_1 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__4; x_2 = lean_alloc_ctor(0, 4, 0); lean_ctor_set(x_2, 0, x_1); lean_ctor_set(x_2, 1, x_1); @@ -65249,13 +65231,13 @@ lean_ctor_set(x_2, 3, x_1); return x_2; } } -static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__13() { +static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__11; -x_2 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__4; -x_3 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__12; +x_1 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__11; +x_2 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__4; +x_3 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__12; x_4 = lean_alloc_ctor(0, 7, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -65267,11 +65249,11 @@ lean_ctor_set(x_4, 6, x_3); return x_4; } } -static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__14() { +static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__14() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__4; +x_1 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__4; x_2 = lean_alloc_ctor(0, 4, 0); lean_ctor_set(x_2, 0, x_1); lean_ctor_set(x_2, 1, x_1); @@ -65280,15 +65262,15 @@ lean_ctor_set(x_2, 3, x_1); return x_2; } } -static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__15() { +static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = lean_box(0); -x_2 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__10; -x_3 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__13; -x_4 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__7; -x_5 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__14; +x_2 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__10; +x_3 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__13; +x_4 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__7; +x_5 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__14; x_6 = lean_alloc_ctor(0, 5, 0); lean_ctor_set(x_6, 0, x_2); lean_ctor_set(x_6, 1, x_3); @@ -65298,7 +65280,7 @@ lean_ctor_set(x_6, 4, x_5); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; uint8_t x_6; @@ -65312,7 +65294,7 @@ x_8 = lean_ctor_get(x_5, 1); x_9 = lean_ctor_get(x_7, 0); lean_inc(x_9); lean_dec(x_7); -x_10 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__1; +x_10 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__1; lean_inc(x_1); x_11 = l_Lean_Tactic_FunInd_isFunInductName(x_9, x_1); lean_dec(x_9); @@ -65336,14 +65318,14 @@ lean_free_object(x_5); x_15 = lean_ctor_get(x_1, 0); lean_inc(x_15); lean_dec(x_1); -x_16 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__15; +x_16 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__15; x_17 = lean_st_mk_ref(x_16, x_8); x_18 = lean_ctor_get(x_17, 0); lean_inc(x_18); x_19 = lean_ctor_get(x_17, 1); lean_inc(x_19); lean_dec(x_17); -x_20 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__9; +x_20 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__9; lean_inc(x_18); x_21 = l_Lean_Tactic_FunInd_deriveInduction(x_15, x_20, x_18, x_2, x_3, x_19); if (lean_obj_tag(x_21) == 0) @@ -65427,7 +65409,7 @@ lean_dec(x_5); x_40 = lean_ctor_get(x_38, 0); lean_inc(x_40); lean_dec(x_38); -x_41 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__1; +x_41 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__1; lean_inc(x_1); x_42 = l_Lean_Tactic_FunInd_isFunInductName(x_40, x_1); lean_dec(x_40); @@ -65449,14 +65431,14 @@ lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean x_46 = lean_ctor_get(x_1, 0); lean_inc(x_46); lean_dec(x_1); -x_47 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__15; +x_47 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__15; x_48 = lean_st_mk_ref(x_47, x_39); x_49 = lean_ctor_get(x_48, 0); lean_inc(x_49); x_50 = lean_ctor_get(x_48, 1); lean_inc(x_50); lean_dec(x_48); -x_51 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__9; +x_51 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__9; lean_inc(x_49); x_52 = l_Lean_Tactic_FunInd_deriveInduction(x_46, x_51, x_49, x_2, x_3, x_50); if (lean_obj_tag(x_52) == 0) @@ -65531,7 +65513,7 @@ return x_66; } } } -static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____closed__1() { +static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____closed__1() { _start: { lean_object* x_1; @@ -65539,19 +65521,19 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_isFunInductName___boxed), return x_1; } } -static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____closed__2() { +static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____closed__2() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2), 4, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2), 4, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____closed__1; +x_2 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____closed__1; x_3 = l_Lean_registerReservedNamePredicate(x_2, x_1); if (lean_obj_tag(x_3) == 0) { @@ -65559,7 +65541,7 @@ lean_object* x_4; lean_object* x_5; lean_object* x_6; x_4 = lean_ctor_get(x_3, 1); lean_inc(x_4); lean_dec(x_3); -x_5 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____closed__2; +x_5 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____closed__2; x_6 = l_Lean_registerReservedNameAction(x_5, x_4); return x_6; } @@ -65587,18 +65569,18 @@ return x_10; } } } -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__1(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__1(x_1, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); return x_5; } } -static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__1() { +static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__1() { _start: { lean_object* x_1; @@ -65606,17 +65588,17 @@ x_1 = lean_mk_string_unchecked("initFn", 6, 6); return x_1; } } -static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__2() { +static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__1; +x_2 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__3() { +static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__3() { _start: { lean_object* x_1; @@ -65624,17 +65606,17 @@ x_1 = lean_mk_string_unchecked("_@", 2, 2); return x_1; } } -static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__4() { +static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__2; -x_2 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__3; +x_1 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__2; +x_2 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__3; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__5() { +static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__5() { _start: { lean_object* x_1; @@ -65642,47 +65624,47 @@ x_1 = lean_mk_string_unchecked("Lean", 4, 4); return x_1; } } -static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__6() { +static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__4; -x_2 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__5; +x_1 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__4; +x_2 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__5; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__7() { +static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__6; +x_1 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__6; x_2 = l_Lean_Tactic_FunInd_buildInductionCase___closed__3; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__8() { +static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__7; +x_1 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__7; x_2 = l_Lean_logAt___at_Lean_Tactic_FunInd_buildInductionBody___spec__41___lambda__2___closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__9() { +static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__8; +x_1 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__8; x_2 = l_Lean_Tactic_FunInd_buildInductionCase___closed__4; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__10() { +static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__10() { _start: { lean_object* x_1; @@ -65690,33 +65672,33 @@ x_1 = lean_mk_string_unchecked("_hyg", 4, 4); return x_1; } } -static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__11() { +static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__9; -x_2 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__10; +x_1 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__9; +x_2 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__10; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__12() { +static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__11; -x_2 = lean_unsigned_to_nat(16616u); +x_1 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__11; +x_2 = lean_unsigned_to_nat(16644u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644_(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; x_2 = l_Lean_Tactic_FunInd_buildInductionCase___closed__5; x_3 = 0; -x_4 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__12; +x_4 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__12; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); return x_5; } @@ -65979,20 +65961,28 @@ l_Lean_Tactic_FunInd_buildInductionBody___lambda__10___closed__1 = _init_l_Lean_ lean_mark_persistent(l_Lean_Tactic_FunInd_buildInductionBody___lambda__10___closed__1); l_Lean_Tactic_FunInd_buildInductionBody___lambda__10___closed__2 = _init_l_Lean_Tactic_FunInd_buildInductionBody___lambda__10___closed__2(); lean_mark_persistent(l_Lean_Tactic_FunInd_buildInductionBody___lambda__10___closed__2); -l_Lean_Tactic_FunInd_buildInductionBody___lambda__19___closed__1 = _init_l_Lean_Tactic_FunInd_buildInductionBody___lambda__19___closed__1(); -lean_mark_persistent(l_Lean_Tactic_FunInd_buildInductionBody___lambda__19___closed__1); -l_Lean_Tactic_FunInd_buildInductionBody___lambda__19___closed__2 = _init_l_Lean_Tactic_FunInd_buildInductionBody___lambda__19___closed__2(); -lean_mark_persistent(l_Lean_Tactic_FunInd_buildInductionBody___lambda__19___closed__2); -l_Lean_Tactic_FunInd_buildInductionBody___lambda__26___closed__1 = _init_l_Lean_Tactic_FunInd_buildInductionBody___lambda__26___closed__1(); -lean_mark_persistent(l_Lean_Tactic_FunInd_buildInductionBody___lambda__26___closed__1); -l_Lean_Tactic_FunInd_buildInductionBody___lambda__26___closed__2 = _init_l_Lean_Tactic_FunInd_buildInductionBody___lambda__26___closed__2(); -lean_mark_persistent(l_Lean_Tactic_FunInd_buildInductionBody___lambda__26___closed__2); +l_Lean_Tactic_FunInd_buildInductionBody___lambda__17___closed__1 = _init_l_Lean_Tactic_FunInd_buildInductionBody___lambda__17___closed__1(); +lean_mark_persistent(l_Lean_Tactic_FunInd_buildInductionBody___lambda__17___closed__1); +l_Lean_Tactic_FunInd_buildInductionBody___lambda__17___closed__2 = _init_l_Lean_Tactic_FunInd_buildInductionBody___lambda__17___closed__2(); +lean_mark_persistent(l_Lean_Tactic_FunInd_buildInductionBody___lambda__17___closed__2); +l_Lean_Tactic_FunInd_buildInductionBody___lambda__17___closed__3 = _init_l_Lean_Tactic_FunInd_buildInductionBody___lambda__17___closed__3(); +lean_mark_persistent(l_Lean_Tactic_FunInd_buildInductionBody___lambda__17___closed__3); +l_Lean_Tactic_FunInd_buildInductionBody___lambda__17___closed__4 = _init_l_Lean_Tactic_FunInd_buildInductionBody___lambda__17___closed__4(); +lean_mark_persistent(l_Lean_Tactic_FunInd_buildInductionBody___lambda__17___closed__4); +l_Lean_Tactic_FunInd_buildInductionBody___lambda__20___closed__1 = _init_l_Lean_Tactic_FunInd_buildInductionBody___lambda__20___closed__1(); +lean_mark_persistent(l_Lean_Tactic_FunInd_buildInductionBody___lambda__20___closed__1); +l_Lean_Tactic_FunInd_buildInductionBody___lambda__20___closed__2 = _init_l_Lean_Tactic_FunInd_buildInductionBody___lambda__20___closed__2(); +lean_mark_persistent(l_Lean_Tactic_FunInd_buildInductionBody___lambda__20___closed__2); +l_Lean_Tactic_FunInd_buildInductionBody___lambda__27___closed__1 = _init_l_Lean_Tactic_FunInd_buildInductionBody___lambda__27___closed__1(); +lean_mark_persistent(l_Lean_Tactic_FunInd_buildInductionBody___lambda__27___closed__1); +l_Lean_Tactic_FunInd_buildInductionBody___lambda__27___closed__2 = _init_l_Lean_Tactic_FunInd_buildInductionBody___lambda__27___closed__2(); +lean_mark_persistent(l_Lean_Tactic_FunInd_buildInductionBody___lambda__27___closed__2); l_Lean_Tactic_FunInd_buildInductionBody___closed__1 = _init_l_Lean_Tactic_FunInd_buildInductionBody___closed__1(); lean_mark_persistent(l_Lean_Tactic_FunInd_buildInductionBody___closed__1); l_Lean_Tactic_FunInd_buildInductionBody___closed__2 = _init_l_Lean_Tactic_FunInd_buildInductionBody___closed__2(); lean_mark_persistent(l_Lean_Tactic_FunInd_buildInductionBody___closed__2); -l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___closed__1 = _init_l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___closed__1(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___closed__1); +l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___closed__1 = _init_l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___closed__1(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___closed__1); l_Lean_Tactic_FunInd_abstractIndependentMVars___lambda__3___closed__1 = _init_l_Lean_Tactic_FunInd_abstractIndependentMVars___lambda__3___closed__1(); lean_mark_persistent(l_Lean_Tactic_FunInd_abstractIndependentMVars___lambda__3___closed__1); l_Lean_Tactic_FunInd_abstractIndependentMVars___lambda__3___closed__2 = _init_l_Lean_Tactic_FunInd_abstractIndependentMVars___lambda__3___closed__2(); @@ -66183,8 +66173,8 @@ l_Lean_Elab_Structural_Positions_groupAndSort___at_Lean_Tactic_FunInd_deriveIndu lean_mark_persistent(l_Lean_Elab_Structural_Positions_groupAndSort___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__3___closed__6); l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__8___closed__1 = _init_l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__8___closed__1(); lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__8___closed__1); -l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9___closed__1 = _init_l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9___closed__1(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9___closed__1); +l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9___closed__1 = _init_l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9___closed__1(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9___closed__1); l_panic___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__13___closed__1 = _init_l_panic___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__13___closed__1(); lean_mark_persistent(l_panic___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__13___closed__1); l_Lean_Elab_Structural_Positions_mapMwith___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__12___closed__1 = _init_l_Lean_Elab_Structural_Positions_mapMwith___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__12___closed__1(); @@ -66321,68 +66311,68 @@ l_Lean_Tactic_FunInd_isFunInductName___lambda__2___closed__1 = _init_l_Lean_Tact lean_mark_persistent(l_Lean_Tactic_FunInd_isFunInductName___lambda__2___closed__1); l_Lean_Tactic_FunInd_isFunInductName___lambda__2___closed__2 = _init_l_Lean_Tactic_FunInd_isFunInductName___lambda__2___closed__2(); lean_mark_persistent(l_Lean_Tactic_FunInd_isFunInductName___lambda__2___closed__2); -l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__1 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__1(); -lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__1); -l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__2 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__2(); -lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__2); -l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__3 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__3(); -lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__3); -l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__4 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__4(); -lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__4); -l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__5 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__5(); -lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__5); -l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__6 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__6(); -lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__6); -l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__7 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__7(); -lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__7); -l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__8 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__8(); -lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__8); -l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__9 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__9(); -lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__9); -l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__10 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__10(); -lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__10); -l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__11 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__11(); -lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__11); -l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__12 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__12(); -lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__12); -l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__13 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__13(); -lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__13); -l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__14 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__14(); -lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__14); -l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__15 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__15(); -lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__15); -l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____closed__1 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____closed__1(); -lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____closed__1); -l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____closed__2 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____closed__2(); -lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____closed__2); -if (builtin) {res = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470_(lean_io_mk_world()); +l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__1 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__1); +l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__2 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__2(); +lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__2); +l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__3 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__3(); +lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__3); +l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__4 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__4(); +lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__4); +l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__5 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__5(); +lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__5); +l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__6 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__6(); +lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__6); +l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__7 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__7(); +lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__7); +l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__8 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__8(); +lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__8); +l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__9 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__9(); +lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__9); +l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__10 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__10(); +lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__10); +l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__11 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__11(); +lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__11); +l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__12 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__12(); +lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__12); +l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__13 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__13(); +lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__13); +l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__14 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__14(); +lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__14); +l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__15 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__15(); +lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____lambda__2___closed__15); +l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____closed__1 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____closed__1(); +lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____closed__1); +l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____closed__2 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____closed__2(); +lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498____closed__2); +if (builtin) {res = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16498_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__1 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__1(); -lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__1); -l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__2 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__2(); -lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__2); -l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__3 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__3(); -lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__3); -l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__4 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__4(); -lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__4); -l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__5 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__5(); -lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__5); -l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__6 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__6(); -lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__6); -l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__7 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__7(); -lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__7); -l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__8 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__8(); -lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__8); -l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__9 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__9(); -lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__9); -l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__10 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__10(); -lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__10); -l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__11 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__11(); -lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__11); -l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__12 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__12(); -lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__12); -if (builtin) {res = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616_(lean_io_mk_world()); +}l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__1 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__1(); +lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__1); +l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__2 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__2(); +lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__2); +l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__3 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__3(); +lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__3); +l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__4 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__4(); +lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__4); +l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__5 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__5(); +lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__5); +l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__6 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__6(); +lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__6); +l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__7 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__7(); +lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__7); +l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__8 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__8(); +lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__8); +l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__9 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__9(); +lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__9); +l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__10 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__10(); +lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__10); +l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__11 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__11(); +lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__11); +l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__12 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__12(); +lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644____closed__12); +if (builtin) {res = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16644_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }return lean_io_result_mk_ok(lean_box(0)); diff --git a/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Nat/Simp.c b/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Nat/Simp.c index 2ae55d3c7f2a..f8cbf25be59b 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Nat/Simp.c +++ b/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Nat/Simp.c @@ -16,73 +16,91 @@ extern "C" { lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); lean_object* l_Lean_mkNatLit(lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___closed__3; +lean_object* l_Lean_mkAppN(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__21; +static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__14; lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); +static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__2; lean_object* l_Lean_Meta_Linear_Nat_toContextExpr(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__9; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__7; static lean_object* l_Lean_Meta_Linear_Nat_simpExpr_x3f___closed__3; static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__7; lean_object* l_Lean_mkAppB(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__10; uint8_t l_Lean_Expr_isAppOfArity(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Linear_Nat_LinearExpr_toExpr(lean_object*); lean_object* l_Lean_Expr_sort___override(lean_object*); +lean_object* lean_array_push(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__15; lean_object* l_Lean_Meta_Linear_Nat_LinearCnstr_toArith(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__15; static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__16; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__3(size_t, size_t, lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpExpr_x3f___closed__1; lean_object* l_Lean_Meta_mkExpectedTypeHint(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_array_fget(lean_object*, lean_object*); lean_object* l_Lean_Meta_Linear_Nat_ToLinear_toLinearCnstr_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___closed__1; static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__19; -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__2; -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__1; -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__3; +LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__5(lean_object*); +static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__3; lean_object* l_Lean_mkApp4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__8; -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__13; +LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_withAbstractAtoms(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_appArg_x21(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_withAbstractAtoms___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkAdd(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkApp6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__8; lean_object* l_Nat_Linear_PolyCnstr_norm(lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__3; uint8_t l_Nat_Linear_PolyCnstr_isUnsat(lean_object*); +static lean_object* l_Lean_Meta_withLocalDecls___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__4___rarg___closed__1; lean_object* l_Lean_Meta_Linear_Nat_ToLinear_run___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_getRevArg_x21(lean_object*, lean_object*); uint8_t lean_expr_eqv(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__23; static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__10; +lean_object* l___private_Lean_CoreM_0__Lean_Core_mkFreshNameImp(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__11; static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__22; +static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__16; static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__5; +static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__2; static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__20; lean_object* l_Lean_Meta_mkEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Linear_Nat_LinearExpr_toArith(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__15; -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__14; lean_object* l_Lean_Meta_mkLE(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Nat_Linear_Poly_toExpr(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_levelZero; static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__12; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__14; lean_object* l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(lean_object*); lean_object* l_List_lengthTRAux___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___closed__4; -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__9; -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__5; -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__18; +LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__5___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__5___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Meta_Linear_Nat_reflTrue; -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__11; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__12; +LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__2(lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__13; lean_object* l_Nat_Linear_Poly_norm(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__3___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__17; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpExpr_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__4; +static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__9; +static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkApp3(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__6; @@ -90,13 +108,25 @@ lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__17; lean_object* l_Nat_Linear_PolyCnstr_toExpr(lean_object*); lean_object* l_Nat_Linear_ExprCnstr_toPoly(lean_object*); -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__7; -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__17; +static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__5; +LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__4(lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); extern lean_object* l_Lean_levelOne; +static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__11; static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__18; lean_object* l_Nat_Linear_Expr_toPoly(lean_object*); +static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__1; static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___closed__5; +static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__3; +static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__1; +lean_object* lean_array_mk(lean_object*); +static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__13; +static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__2; +lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_SynthInstance_removeUnusedArguments_x3f___spec__2___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__4; +size_t lean_usize_add(size_t, size_t); +lean_object* lean_array_uget(lean_object*, size_t); +size_t lean_array_size(lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__4; static lean_object* l_Lean_Meta_Linear_Nat_simpExpr_x3f___closed__2; static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___closed__6; @@ -104,12 +134,18 @@ static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___closed__2 lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Nat_Linear_PolyCnstr_isValid(lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__8; -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__16; +lean_object* lean_array_get_size(lean_object*); +static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__10; +static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__1; +uint8_t lean_usize_dec_lt(size_t, size_t); +lean_object* l_Lean_Meta_mkLambdaFVars(lean_object*, lean_object*, uint8_t, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__3; lean_object* l_Lean_Meta_Linear_Nat_ToLinear_toLinearExpr(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__2; -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__6; -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__12; -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__1() { +lean_object* l_Lean_Expr_beta(lean_object*, lean_object*); +lean_object* lean_array_uset(lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__1() { _start: { lean_object* x_1; @@ -117,83 +153,907 @@ x_1 = lean_mk_string_unchecked("Nat", 3, 3); return x_1; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__2() { +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Linear", 6, 6); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} } +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__2; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__3() { +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; +x_7 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__3; +x_8 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_8, 0, x_7); +lean_ctor_set(x_8, 1, x_6); +return x_8; +} +} +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("ExprCnstr", 9, 9); +x_1 = lean_mk_string_unchecked("x", 1, 1); return x_1; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__4() { +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__3() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("eq_of_toNormPoly_eq", 19, 19); +x_1 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___boxed), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__5() { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1(size_t x_1, size_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__1; -x_2 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__2; -x_3 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__3; -x_4 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__4; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; +uint8_t x_9; +x_9 = lean_usize_dec_lt(x_2, x_1); +if (x_9 == 0) +{ +lean_object* x_10; +x_10 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_10, 0, x_3); +lean_ctor_set(x_10, 1, x_8); +return x_10; } +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_11 = lean_unsigned_to_nat(0u); +x_12 = lean_array_uset(x_3, x_2, x_11); +x_13 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__2; +x_14 = l___private_Lean_CoreM_0__Lean_Core_mkFreshNameImp(x_13, x_6, x_7, x_8); +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 0) +{ +lean_object* x_16; lean_object* x_17; size_t x_18; size_t x_19; lean_object* x_20; +x_16 = lean_ctor_get(x_14, 1); +x_17 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__3; +lean_ctor_set(x_14, 1, x_17); +x_18 = 1; +x_19 = lean_usize_add(x_2, x_18); +x_20 = lean_array_uset(x_12, x_2, x_14); +x_2 = x_19; +x_3 = x_20; +x_8 = x_16; +goto _start; } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__6() { +else +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; size_t x_26; size_t x_27; lean_object* x_28; +x_22 = lean_ctor_get(x_14, 0); +x_23 = lean_ctor_get(x_14, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_14); +x_24 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__3; +x_25 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_25, 0, x_22); +lean_ctor_set(x_25, 1, x_24); +x_26 = 1; +x_27 = lean_usize_add(x_2, x_26); +x_28 = lean_array_uset(x_12, x_2, x_25); +x_2 = x_27; +x_3 = x_28; +x_8 = x_23; +goto _start; +} +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__3(size_t x_1, size_t x_2, lean_object* x_3) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__5; -x_3 = l_Lean_Expr_const___override(x_2, x_1); +uint8_t x_4; +x_4 = lean_usize_dec_lt(x_2, x_1); +if (x_4 == 0) +{ return x_3; } +else +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; size_t x_8; size_t x_9; uint8_t x_10; +x_5 = lean_array_uget(x_3, x_2); +x_6 = lean_unsigned_to_nat(0u); +x_7 = lean_array_uset(x_3, x_2, x_6); +x_8 = 1; +x_9 = lean_usize_add(x_2, x_8); +x_10 = !lean_is_exclusive(x_5); +if (x_10 == 0) +{ +lean_object* x_11; uint8_t x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_11 = lean_ctor_get(x_5, 0); +x_12 = 0; +x_13 = lean_box(x_12); +lean_ctor_set(x_5, 0, x_13); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_11); +lean_ctor_set(x_14, 1, x_5); +x_15 = lean_array_uset(x_7, x_2, x_14); +x_2 = x_9; +x_3 = x_15; +goto _start; +} +else +{ +lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_17 = lean_ctor_get(x_5, 0); +x_18 = lean_ctor_get(x_5, 1); +lean_inc(x_18); +lean_inc(x_17); +lean_dec(x_5); +x_19 = 0; +x_20 = lean_box(x_19); +x_21 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_21, 0, x_20); +lean_ctor_set(x_21, 1, x_18); +x_22 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_22, 0, x_17); +lean_ctor_set(x_22, 1, x_21); +x_23 = lean_array_uset(x_7, x_2, x_22); +x_2 = x_9; +x_3 = x_23; +goto _start; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__5___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; +x_11 = lean_array_push(x_1, x_5); +x_12 = l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__5___rarg(x_2, x_3, x_4, x_11, x_6, x_7, x_8, x_9, x_10); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__5___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; uint8_t x_12; +x_10 = lean_array_get_size(x_4); +x_11 = lean_array_get_size(x_1); +x_12 = lean_nat_dec_lt(x_10, x_11); +lean_dec(x_11); +if (x_12 == 0) +{ +lean_object* x_13; +lean_dec(x_10); +lean_dec(x_3); +lean_dec(x_1); +x_13 = lean_apply_6(x_2, x_4, x_5, x_6, x_7, x_8, x_9); +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_14 = lean_array_fget(x_1, x_10); +lean_dec(x_10); +x_15 = lean_ctor_get(x_14, 1); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 0); +lean_inc(x_16); +lean_dec(x_14); +x_17 = lean_ctor_get(x_15, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_15, 1); +lean_inc(x_18); +lean_dec(x_15); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_19 = lean_apply_6(x_18, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_19) == 0) +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; uint8_t x_24; lean_object* x_25; +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_19, 1); +lean_inc(x_21); +lean_dec(x_19); +x_22 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__5___rarg___lambda__1), 10, 4); +lean_closure_set(x_22, 0, x_4); +lean_closure_set(x_22, 1, x_1); +lean_closure_set(x_22, 2, x_2); +lean_closure_set(x_22, 3, x_3); +x_23 = 0; +x_24 = lean_unbox(x_17); +lean_dec(x_17); +x_25 = l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_SynthInstance_removeUnusedArguments_x3f___spec__2___rarg(x_16, x_24, x_20, x_22, x_23, x_5, x_6, x_7, x_8, x_21); +return x_25; +} +else +{ +uint8_t x_26; +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_26 = !lean_is_exclusive(x_19); +if (x_26 == 0) +{ +return x_19; +} +else +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_19, 0); +x_28 = lean_ctor_get(x_19, 1); +lean_inc(x_28); +lean_inc(x_27); +lean_dec(x_19); +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_27); +lean_ctor_set(x_29, 1, x_28); +return x_29; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__5(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__5___rarg), 9, 0); +return x_2; +} +} +static lean_object* _init_l_Lean_Meta_withLocalDecls___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__4___rarg___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_array_mk(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__4___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; lean_object* x_10; +x_9 = l_Lean_Meta_withLocalDecls___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__4___rarg___closed__1; +x_10 = l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__5___rarg(x_2, x_3, x_1, x_9, x_4, x_5, x_6, x_7, x_8); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__4(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecls___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__4___rarg), 8, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +size_t x_9; size_t x_10; lean_object* x_11; lean_object* x_12; +x_9 = lean_array_size(x_2); +x_10 = 0; +x_11 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__3(x_9, x_10, x_2); +x_12 = l_Lean_Meta_withLocalDecls___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__4___rarg(x_1, x_11, x_3, x_4, x_5, x_6, x_7, x_8); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__2(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__2___rarg), 8, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_withAbstractAtoms___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_10 = lean_apply_6(x_1, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_10) == 0) +{ +lean_object* x_11; +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +if (lean_obj_tag(x_11) == 0) +{ +uint8_t x_12; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_12 = !lean_is_exclusive(x_10); +if (x_12 == 0) +{ +lean_object* x_13; +x_13 = lean_ctor_get(x_10, 0); +lean_dec(x_13); +lean_ctor_set(x_10, 0, x_2); +return x_10; +} +else +{ +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_10, 1); +lean_inc(x_14); +lean_dec(x_10); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_2); +lean_ctor_set(x_15, 1, x_14); +return x_15; +} +} +else +{ +uint8_t x_16; +lean_dec(x_2); +x_16 = !lean_is_exclusive(x_11); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; uint8_t x_19; +x_17 = lean_ctor_get(x_11, 0); +x_18 = lean_ctor_get(x_10, 1); +lean_inc(x_18); +lean_dec(x_10); +x_19 = !lean_is_exclusive(x_17); +if (x_19 == 0) +{ +lean_object* x_20; lean_object* x_21; uint8_t x_22; uint8_t x_23; uint8_t x_24; lean_object* x_25; +x_20 = lean_ctor_get(x_17, 0); +x_21 = lean_ctor_get(x_17, 1); +x_22 = 0; +x_23 = 1; +x_24 = 1; +lean_inc(x_4); +x_25 = l_Lean_Meta_mkLambdaFVars(x_4, x_20, x_22, x_23, x_22, x_24, x_5, x_6, x_7, x_8, x_18); +if (lean_obj_tag(x_25) == 0) +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_26 = lean_ctor_get(x_25, 0); +lean_inc(x_26); +x_27 = lean_ctor_get(x_25, 1); +lean_inc(x_27); +lean_dec(x_25); +lean_inc(x_3); +x_28 = l_Lean_Expr_beta(x_26, x_3); +x_29 = l_Lean_Meta_mkLambdaFVars(x_4, x_21, x_22, x_23, x_22, x_24, x_5, x_6, x_7, x_8, x_27); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +if (lean_obj_tag(x_29) == 0) +{ +uint8_t x_30; +x_30 = !lean_is_exclusive(x_29); +if (x_30 == 0) +{ +lean_object* x_31; lean_object* x_32; +x_31 = lean_ctor_get(x_29, 0); +x_32 = l_Lean_mkAppN(x_31, x_3); +lean_dec(x_3); +lean_ctor_set(x_17, 1, x_32); +lean_ctor_set(x_17, 0, x_28); +lean_ctor_set(x_29, 0, x_11); +return x_29; +} +else +{ +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_33 = lean_ctor_get(x_29, 0); +x_34 = lean_ctor_get(x_29, 1); +lean_inc(x_34); +lean_inc(x_33); +lean_dec(x_29); +x_35 = l_Lean_mkAppN(x_33, x_3); +lean_dec(x_3); +lean_ctor_set(x_17, 1, x_35); +lean_ctor_set(x_17, 0, x_28); +x_36 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_36, 0, x_11); +lean_ctor_set(x_36, 1, x_34); +return x_36; +} +} +else +{ +uint8_t x_37; +lean_dec(x_28); +lean_free_object(x_17); +lean_free_object(x_11); +lean_dec(x_3); +x_37 = !lean_is_exclusive(x_29); +if (x_37 == 0) +{ +return x_29; +} +else +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_29, 0); +x_39 = lean_ctor_get(x_29, 1); +lean_inc(x_39); +lean_inc(x_38); +lean_dec(x_29); +x_40 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +return x_40; +} +} +} +else +{ +uint8_t x_41; +lean_free_object(x_17); +lean_dec(x_21); +lean_free_object(x_11); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_41 = !lean_is_exclusive(x_25); +if (x_41 == 0) +{ +return x_25; +} +else +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_42 = lean_ctor_get(x_25, 0); +x_43 = lean_ctor_get(x_25, 1); +lean_inc(x_43); +lean_inc(x_42); +lean_dec(x_25); +x_44 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_44, 0, x_42); +lean_ctor_set(x_44, 1, x_43); +return x_44; +} +} +} +else +{ +lean_object* x_45; lean_object* x_46; uint8_t x_47; uint8_t x_48; uint8_t x_49; lean_object* x_50; +x_45 = lean_ctor_get(x_17, 0); +x_46 = lean_ctor_get(x_17, 1); +lean_inc(x_46); +lean_inc(x_45); +lean_dec(x_17); +x_47 = 0; +x_48 = 1; +x_49 = 1; +lean_inc(x_4); +x_50 = l_Lean_Meta_mkLambdaFVars(x_4, x_45, x_47, x_48, x_47, x_49, x_5, x_6, x_7, x_8, x_18); +if (lean_obj_tag(x_50) == 0) +{ +lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_51 = lean_ctor_get(x_50, 0); +lean_inc(x_51); +x_52 = lean_ctor_get(x_50, 1); +lean_inc(x_52); +lean_dec(x_50); +lean_inc(x_3); +x_53 = l_Lean_Expr_beta(x_51, x_3); +x_54 = l_Lean_Meta_mkLambdaFVars(x_4, x_46, x_47, x_48, x_47, x_49, x_5, x_6, x_7, x_8, x_52); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +if (lean_obj_tag(x_54) == 0) +{ +lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; +x_55 = lean_ctor_get(x_54, 0); +lean_inc(x_55); +x_56 = lean_ctor_get(x_54, 1); +lean_inc(x_56); +if (lean_is_exclusive(x_54)) { + lean_ctor_release(x_54, 0); + lean_ctor_release(x_54, 1); + x_57 = x_54; +} else { + lean_dec_ref(x_54); + x_57 = lean_box(0); +} +x_58 = l_Lean_mkAppN(x_55, x_3); +lean_dec(x_3); +x_59 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_59, 0, x_53); +lean_ctor_set(x_59, 1, x_58); +lean_ctor_set(x_11, 0, x_59); +if (lean_is_scalar(x_57)) { + x_60 = lean_alloc_ctor(0, 2, 0); +} else { + x_60 = x_57; +} +lean_ctor_set(x_60, 0, x_11); +lean_ctor_set(x_60, 1, x_56); +return x_60; +} +else +{ +lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; +lean_dec(x_53); +lean_free_object(x_11); +lean_dec(x_3); +x_61 = lean_ctor_get(x_54, 0); +lean_inc(x_61); +x_62 = lean_ctor_get(x_54, 1); +lean_inc(x_62); +if (lean_is_exclusive(x_54)) { + lean_ctor_release(x_54, 0); + lean_ctor_release(x_54, 1); + x_63 = x_54; +} else { + lean_dec_ref(x_54); + x_63 = lean_box(0); +} +if (lean_is_scalar(x_63)) { + x_64 = lean_alloc_ctor(1, 2, 0); +} else { + x_64 = x_63; +} +lean_ctor_set(x_64, 0, x_61); +lean_ctor_set(x_64, 1, x_62); +return x_64; +} +} +else +{ +lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; +lean_dec(x_46); +lean_free_object(x_11); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_65 = lean_ctor_get(x_50, 0); +lean_inc(x_65); +x_66 = lean_ctor_get(x_50, 1); +lean_inc(x_66); +if (lean_is_exclusive(x_50)) { + lean_ctor_release(x_50, 0); + lean_ctor_release(x_50, 1); + x_67 = x_50; +} else { + lean_dec_ref(x_50); + x_67 = lean_box(0); +} +if (lean_is_scalar(x_67)) { + x_68 = lean_alloc_ctor(1, 2, 0); +} else { + x_68 = x_67; +} +lean_ctor_set(x_68, 0, x_65); +lean_ctor_set(x_68, 1, x_66); +return x_68; +} +} +} +else +{ +lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; uint8_t x_74; uint8_t x_75; uint8_t x_76; lean_object* x_77; +x_69 = lean_ctor_get(x_11, 0); +lean_inc(x_69); +lean_dec(x_11); +x_70 = lean_ctor_get(x_10, 1); +lean_inc(x_70); +lean_dec(x_10); +x_71 = lean_ctor_get(x_69, 0); +lean_inc(x_71); +x_72 = lean_ctor_get(x_69, 1); +lean_inc(x_72); +if (lean_is_exclusive(x_69)) { + lean_ctor_release(x_69, 0); + lean_ctor_release(x_69, 1); + x_73 = x_69; +} else { + lean_dec_ref(x_69); + x_73 = lean_box(0); +} +x_74 = 0; +x_75 = 1; +x_76 = 1; +lean_inc(x_4); +x_77 = l_Lean_Meta_mkLambdaFVars(x_4, x_71, x_74, x_75, x_74, x_76, x_5, x_6, x_7, x_8, x_70); +if (lean_obj_tag(x_77) == 0) +{ +lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_78 = lean_ctor_get(x_77, 0); +lean_inc(x_78); +x_79 = lean_ctor_get(x_77, 1); +lean_inc(x_79); +lean_dec(x_77); +lean_inc(x_3); +x_80 = l_Lean_Expr_beta(x_78, x_3); +x_81 = l_Lean_Meta_mkLambdaFVars(x_4, x_72, x_74, x_75, x_74, x_76, x_5, x_6, x_7, x_8, x_79); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +if (lean_obj_tag(x_81) == 0) +{ +lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; +x_82 = lean_ctor_get(x_81, 0); +lean_inc(x_82); +x_83 = lean_ctor_get(x_81, 1); +lean_inc(x_83); +if (lean_is_exclusive(x_81)) { + lean_ctor_release(x_81, 0); + lean_ctor_release(x_81, 1); + x_84 = x_81; +} else { + lean_dec_ref(x_81); + x_84 = lean_box(0); +} +x_85 = l_Lean_mkAppN(x_82, x_3); +lean_dec(x_3); +if (lean_is_scalar(x_73)) { + x_86 = lean_alloc_ctor(0, 2, 0); +} else { + x_86 = x_73; +} +lean_ctor_set(x_86, 0, x_80); +lean_ctor_set(x_86, 1, x_85); +x_87 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_87, 0, x_86); +if (lean_is_scalar(x_84)) { + x_88 = lean_alloc_ctor(0, 2, 0); +} else { + x_88 = x_84; +} +lean_ctor_set(x_88, 0, x_87); +lean_ctor_set(x_88, 1, x_83); +return x_88; +} +else +{ +lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; +lean_dec(x_80); +lean_dec(x_73); +lean_dec(x_3); +x_89 = lean_ctor_get(x_81, 0); +lean_inc(x_89); +x_90 = lean_ctor_get(x_81, 1); +lean_inc(x_90); +if (lean_is_exclusive(x_81)) { + lean_ctor_release(x_81, 0); + lean_ctor_release(x_81, 1); + x_91 = x_81; +} else { + lean_dec_ref(x_81); + x_91 = lean_box(0); } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__7() { +if (lean_is_scalar(x_91)) { + x_92 = lean_alloc_ctor(1, 2, 0); +} else { + x_92 = x_91; +} +lean_ctor_set(x_92, 0, x_89); +lean_ctor_set(x_92, 1, x_90); +return x_92; +} +} +else +{ +lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; +lean_dec(x_73); +lean_dec(x_72); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_93 = lean_ctor_get(x_77, 0); +lean_inc(x_93); +x_94 = lean_ctor_get(x_77, 1); +lean_inc(x_94); +if (lean_is_exclusive(x_77)) { + lean_ctor_release(x_77, 0); + lean_ctor_release(x_77, 1); + x_95 = x_77; +} else { + lean_dec_ref(x_77); + x_95 = lean_box(0); +} +if (lean_is_scalar(x_95)) { + x_96 = lean_alloc_ctor(1, 2, 0); +} else { + x_96 = x_95; +} +lean_ctor_set(x_96, 0, x_93); +lean_ctor_set(x_96, 1, x_94); +return x_96; +} +} +} +} +else +{ +uint8_t x_97; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_97 = !lean_is_exclusive(x_10); +if (x_97 == 0) +{ +return x_10; +} +else +{ +lean_object* x_98; lean_object* x_99; lean_object* x_100; +x_98 = lean_ctor_get(x_10, 0); +x_99 = lean_ctor_get(x_10, 1); +lean_inc(x_99); +lean_inc(x_98); +lean_dec(x_10); +x_100 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_100, 0, x_98); +lean_ctor_set(x_100, 1, x_99); +return x_100; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_withAbstractAtoms(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +size_t x_8; size_t x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_8 = lean_array_size(x_1); +x_9 = 0; +lean_inc(x_1); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1(x_8, x_9, x_1, x_3, x_4, x_5, x_6, x_7); +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_10, 1); +lean_inc(x_12); +lean_dec(x_10); +x_13 = lean_box(0); +x_14 = lean_alloc_closure((void*)(l_Lean_Meta_Linear_Nat_withAbstractAtoms___lambda__1), 9, 3); +lean_closure_set(x_14, 0, x_2); +lean_closure_set(x_14, 1, x_13); +lean_closure_set(x_14, 2, x_1); +x_15 = l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__2___rarg(x_13, x_11, x_14, x_3, x_4, x_5, x_6, x_12); +return x_15; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; +x_7 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +size_t x_9; size_t x_10; lean_object* x_11; +x_9 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_10 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_11 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1(x_9, x_10, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; size_t x_5; lean_object* x_6; +x_4 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__3(x_4, x_5, x_3); +return x_6; +} +} +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("eq_true_of_isValid", 18, 18); +x_1 = lean_mk_string_unchecked("Linear", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("ExprCnstr", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__8() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("eq_of_toNormPoly_eq", 19, 19); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__1; -x_2 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__2; -x_3 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__3; -x_4 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__7; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__1; +x_2 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__1; +x_3 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__2; +x_4 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__3; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__9() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__8; +x_2 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__4; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__10() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__6() { _start: { lean_object* x_1; @@ -201,57 +1061,57 @@ x_1 = lean_mk_string_unchecked("True", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__11() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__10; +x_2 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__12() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__11; +x_2 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__7; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__13() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__9() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("eq_false_of_isUnsat", 19, 19); +x_1 = lean_mk_string_unchecked("eq_true_of_isValid", 18, 18); return x_1; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__14() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__1; -x_2 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__2; -x_3 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__3; -x_4 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__13; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__1; +x_2 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__1; +x_3 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__2; +x_4 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__9; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__15() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__14; +x_2 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__10; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__16() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__12() { _start: { lean_object* x_1; @@ -259,381 +1119,418 @@ x_1 = lean_mk_string_unchecked("False", 5, 5); return x_1; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__17() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__16; +x_2 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__12; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__18() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__17; +x_2 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__13; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__15() { _start: { -lean_object* x_7; lean_object* x_8; -lean_inc(x_1); -x_7 = lean_alloc_closure((void*)(l_Lean_Meta_Linear_Nat_ToLinear_toLinearCnstr_x3f), 7, 1); -lean_closure_set(x_7, 0, x_1); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_2); -x_8 = l_Lean_Meta_Linear_Nat_ToLinear_run___rarg(x_7, x_2, x_3, x_4, x_5, x_6); -if (lean_obj_tag(x_8) == 0) -{ -lean_object* x_9; lean_object* x_10; -x_9 = lean_ctor_get(x_8, 0); -lean_inc(x_9); -x_10 = lean_ctor_get(x_9, 0); -lean_inc(x_10); -if (lean_obj_tag(x_10) == 0) -{ -uint8_t x_11; -lean_dec(x_9); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_11 = !lean_is_exclusive(x_8); -if (x_11 == 0) -{ -lean_object* x_12; lean_object* x_13; -x_12 = lean_ctor_get(x_8, 0); -lean_dec(x_12); -x_13 = lean_box(0); -lean_ctor_set(x_8, 0, x_13); -return x_8; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("eq_false_of_isUnsat", 19, 19); +return x_1; } -else +} +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__16() { +_start: { -lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_14 = lean_ctor_get(x_8, 1); -lean_inc(x_14); -lean_dec(x_8); -x_15 = lean_box(0); -x_16 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_16, 0, x_15); -lean_ctor_set(x_16, 1, x_14); -return x_16; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__1; +x_2 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__1; +x_3 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__2; +x_4 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__15; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; } } -else +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__17() { +_start: { -lean_object* x_17; uint8_t x_18; -x_17 = lean_ctor_get(x_8, 1); -lean_inc(x_17); -lean_dec(x_8); -x_18 = !lean_is_exclusive(x_9); -if (x_18 == 0) +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__16; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: { -lean_object* x_19; lean_object* x_20; uint8_t x_21; -x_19 = lean_ctor_get(x_9, 1); -x_20 = lean_ctor_get(x_9, 0); -lean_dec(x_20); -x_21 = !lean_is_exclusive(x_10); -if (x_21 == 0) +lean_object* x_8; uint8_t x_9; +lean_inc(x_1); +x_8 = l_Lean_Meta_Linear_Nat_LinearCnstr_toArith(x_2, x_1, x_3, x_4, x_5, x_6, x_7); +x_9 = !lean_is_exclusive(x_8); +if (x_9 == 0) { -lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; -x_22 = lean_ctor_get(x_10, 0); -lean_inc(x_22); -x_23 = l_Nat_Linear_ExprCnstr_toPoly(x_22); -x_24 = l_Nat_Linear_PolyCnstr_norm(x_23); -x_25 = l_Nat_Linear_PolyCnstr_isUnsat(x_24); -if (x_25 == 0) +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_10 = lean_ctor_get(x_8, 0); +x_11 = lean_ctor_get(x_8, 1); +lean_inc(x_1); +x_12 = l_Nat_Linear_ExprCnstr_toPoly(x_1); +x_13 = l_Nat_Linear_PolyCnstr_norm(x_12); +x_14 = l_Nat_Linear_PolyCnstr_isUnsat(x_13); +if (x_14 == 0) { -uint8_t x_26; -x_26 = l_Nat_Linear_PolyCnstr_isValid(x_24); -if (x_26 == 0) +uint8_t x_15; +x_15 = l_Nat_Linear_PolyCnstr_isValid(x_13); +if (x_15 == 0) { -lean_object* x_27; lean_object* x_28; uint8_t x_29; -x_27 = l_Nat_Linear_PolyCnstr_toExpr(x_24); -lean_inc(x_27); -x_28 = l_Lean_Meta_Linear_Nat_LinearCnstr_toArith(x_19, x_27, x_2, x_3, x_4, x_5, x_17); -x_29 = !lean_is_exclusive(x_28); -if (x_29 == 0) -{ -lean_object* x_30; lean_object* x_31; uint8_t x_32; -x_30 = lean_ctor_get(x_28, 0); -x_31 = lean_ctor_get(x_28, 1); -x_32 = lean_expr_eqv(x_30, x_1); -if (x_32 == 0) +lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_16 = l_Nat_Linear_PolyCnstr_toExpr(x_13); +lean_inc(x_16); +x_17 = l_Lean_Meta_Linear_Nat_LinearCnstr_toArith(x_2, x_16, x_3, x_4, x_5, x_6, x_11); +x_18 = !lean_is_exclusive(x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_19 = lean_ctor_get(x_17, 0); +x_20 = lean_ctor_get(x_17, 1); +x_21 = lean_expr_eqv(x_19, x_10); +if (x_21 == 0) { -lean_object* x_33; -lean_free_object(x_28); +lean_object* x_22; +lean_free_object(x_17); +lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -lean_inc(x_2); -x_33 = l_Lean_Meta_Linear_Nat_toContextExpr(x_19, x_2, x_3, x_4, x_5, x_31); -if (lean_obj_tag(x_33) == 0) +x_22 = l_Lean_Meta_Linear_Nat_toContextExpr(x_2, x_3, x_4, x_5, x_6, x_20); +if (lean_obj_tag(x_22) == 0) { -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_34 = lean_ctor_get(x_33, 0); -lean_inc(x_34); -x_35 = lean_ctor_get(x_33, 1); -lean_inc(x_35); -lean_dec(x_33); -x_36 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_22); -x_37 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_27); -x_38 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__6; -x_39 = l_Lean_Meta_Linear_Nat_reflTrue; -x_40 = l_Lean_mkApp4(x_38, x_34, x_36, x_37, x_39); +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +lean_dec(x_22); +x_25 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_1); +x_26 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_16); +x_27 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__5; +x_28 = l_Lean_Meta_Linear_Nat_reflTrue; +x_29 = l_Lean_mkApp4(x_27, x_23, x_25, x_26, x_28); +lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -lean_inc(x_2); -lean_inc(x_30); -x_41 = l_Lean_Meta_mkEq(x_1, x_30, x_2, x_3, x_4, x_5, x_35); -if (lean_obj_tag(x_41) == 0) -{ -lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_ctor_get(x_41, 0); -lean_inc(x_42); -x_43 = lean_ctor_get(x_41, 1); -lean_inc(x_43); -lean_dec(x_41); -x_44 = l_Lean_Meta_mkExpectedTypeHint(x_40, x_42, x_2, x_3, x_4, x_5, x_43); -if (lean_obj_tag(x_44) == 0) +lean_inc(x_19); +x_30 = l_Lean_Meta_mkEq(x_10, x_19, x_3, x_4, x_5, x_6, x_24); +if (lean_obj_tag(x_30) == 0) { -uint8_t x_45; -x_45 = !lean_is_exclusive(x_44); -if (x_45 == 0) +lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_31 = lean_ctor_get(x_30, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_30, 1); +lean_inc(x_32); +lean_dec(x_30); +x_33 = l_Lean_Meta_mkExpectedTypeHint(x_29, x_31, x_3, x_4, x_5, x_6, x_32); +if (lean_obj_tag(x_33) == 0) { -lean_object* x_46; -x_46 = lean_ctor_get(x_44, 0); -lean_ctor_set(x_9, 1, x_46); -lean_ctor_set(x_9, 0, x_30); -lean_ctor_set(x_10, 0, x_9); -lean_ctor_set(x_44, 0, x_10); -return x_44; +uint8_t x_34; +x_34 = !lean_is_exclusive(x_33); +if (x_34 == 0) +{ +lean_object* x_35; lean_object* x_36; +x_35 = lean_ctor_get(x_33, 0); +lean_ctor_set(x_8, 1, x_35); +lean_ctor_set(x_8, 0, x_19); +x_36 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_36, 0, x_8); +lean_ctor_set(x_33, 0, x_36); +return x_33; } else { -lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_47 = lean_ctor_get(x_44, 0); -x_48 = lean_ctor_get(x_44, 1); -lean_inc(x_48); -lean_inc(x_47); -lean_dec(x_44); -lean_ctor_set(x_9, 1, x_47); -lean_ctor_set(x_9, 0, x_30); -lean_ctor_set(x_10, 0, x_9); -x_49 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_49, 0, x_10); -lean_ctor_set(x_49, 1, x_48); -return x_49; +lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_37 = lean_ctor_get(x_33, 0); +x_38 = lean_ctor_get(x_33, 1); +lean_inc(x_38); +lean_inc(x_37); +lean_dec(x_33); +lean_ctor_set(x_8, 1, x_37); +lean_ctor_set(x_8, 0, x_19); +x_39 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_39, 0, x_8); +x_40 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_40, 0, x_39); +lean_ctor_set(x_40, 1, x_38); +return x_40; } } else { -uint8_t x_50; -lean_dec(x_30); -lean_free_object(x_10); -lean_free_object(x_9); -x_50 = !lean_is_exclusive(x_44); -if (x_50 == 0) +uint8_t x_41; +lean_dec(x_19); +lean_free_object(x_8); +x_41 = !lean_is_exclusive(x_33); +if (x_41 == 0) { -return x_44; +return x_33; } else { -lean_object* x_51; lean_object* x_52; lean_object* x_53; -x_51 = lean_ctor_get(x_44, 0); -x_52 = lean_ctor_get(x_44, 1); -lean_inc(x_52); -lean_inc(x_51); -lean_dec(x_44); -x_53 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_53, 0, x_51); -lean_ctor_set(x_53, 1, x_52); -return x_53; +lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_42 = lean_ctor_get(x_33, 0); +x_43 = lean_ctor_get(x_33, 1); +lean_inc(x_43); +lean_inc(x_42); +lean_dec(x_33); +x_44 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_44, 0, x_42); +lean_ctor_set(x_44, 1, x_43); +return x_44; } } } else { -uint8_t x_54; -lean_dec(x_40); -lean_dec(x_30); -lean_free_object(x_10); -lean_free_object(x_9); +uint8_t x_45; +lean_dec(x_29); +lean_dec(x_19); +lean_free_object(x_8); +lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); -x_54 = !lean_is_exclusive(x_41); -if (x_54 == 0) +x_45 = !lean_is_exclusive(x_30); +if (x_45 == 0) { -return x_41; +return x_30; } else { -lean_object* x_55; lean_object* x_56; lean_object* x_57; -x_55 = lean_ctor_get(x_41, 0); -x_56 = lean_ctor_get(x_41, 1); -lean_inc(x_56); -lean_inc(x_55); -lean_dec(x_41); -x_57 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_57, 0, x_55); -lean_ctor_set(x_57, 1, x_56); -return x_57; +lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_46 = lean_ctor_get(x_30, 0); +x_47 = lean_ctor_get(x_30, 1); +lean_inc(x_47); +lean_inc(x_46); +lean_dec(x_30); +x_48 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_48, 0, x_46); +lean_ctor_set(x_48, 1, x_47); +return x_48; } } } else { -uint8_t x_58; -lean_dec(x_30); -lean_dec(x_27); -lean_free_object(x_10); -lean_dec(x_22); -lean_free_object(x_9); +uint8_t x_49; +lean_dec(x_19); +lean_dec(x_16); +lean_free_object(x_8); +lean_dec(x_10); +lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); lean_dec(x_1); -x_58 = !lean_is_exclusive(x_33); -if (x_58 == 0) +x_49 = !lean_is_exclusive(x_22); +if (x_49 == 0) { -return x_33; +return x_22; } else { -lean_object* x_59; lean_object* x_60; lean_object* x_61; -x_59 = lean_ctor_get(x_33, 0); -x_60 = lean_ctor_get(x_33, 1); -lean_inc(x_60); -lean_inc(x_59); -lean_dec(x_33); -x_61 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_61, 0, x_59); -lean_ctor_set(x_61, 1, x_60); -return x_61; +lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_50 = lean_ctor_get(x_22, 0); +x_51 = lean_ctor_get(x_22, 1); +lean_inc(x_51); +lean_inc(x_50); +lean_dec(x_22); +x_52 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_52, 0, x_50); +lean_ctor_set(x_52, 1, x_51); +return x_52; } } } else { -lean_object* x_62; -lean_dec(x_30); -lean_dec(x_27); -lean_free_object(x_10); -lean_dec(x_22); -lean_free_object(x_9); +lean_object* x_53; lean_dec(x_19); +lean_dec(x_16); +lean_free_object(x_8); +lean_dec(x_10); +lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_62 = lean_box(0); -lean_ctor_set(x_28, 0, x_62); -return x_28; +x_53 = lean_box(0); +lean_ctor_set(x_17, 0, x_53); +return x_17; } } else { -lean_object* x_63; lean_object* x_64; uint8_t x_65; -x_63 = lean_ctor_get(x_28, 0); -x_64 = lean_ctor_get(x_28, 1); -lean_inc(x_64); -lean_inc(x_63); -lean_dec(x_28); -x_65 = lean_expr_eqv(x_63, x_1); -if (x_65 == 0) +lean_object* x_54; lean_object* x_55; uint8_t x_56; +x_54 = lean_ctor_get(x_17, 0); +x_55 = lean_ctor_get(x_17, 1); +lean_inc(x_55); +lean_inc(x_54); +lean_dec(x_17); +x_56 = lean_expr_eqv(x_54, x_10); +if (x_56 == 0) { -lean_object* x_66; +lean_object* x_57; +lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -lean_inc(x_2); -x_66 = l_Lean_Meta_Linear_Nat_toContextExpr(x_19, x_2, x_3, x_4, x_5, x_64); -if (lean_obj_tag(x_66) == 0) +x_57 = l_Lean_Meta_Linear_Nat_toContextExpr(x_2, x_3, x_4, x_5, x_6, x_55); +if (lean_obj_tag(x_57) == 0) { -lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; -x_67 = lean_ctor_get(x_66, 0); -lean_inc(x_67); -x_68 = lean_ctor_get(x_66, 1); -lean_inc(x_68); -lean_dec(x_66); -x_69 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_22); -x_70 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_27); -x_71 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__6; -x_72 = l_Lean_Meta_Linear_Nat_reflTrue; -x_73 = l_Lean_mkApp4(x_71, x_67, x_69, x_70, x_72); +lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_58 = lean_ctor_get(x_57, 0); +lean_inc(x_58); +x_59 = lean_ctor_get(x_57, 1); +lean_inc(x_59); +lean_dec(x_57); +x_60 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_1); +x_61 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_16); +x_62 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__5; +x_63 = l_Lean_Meta_Linear_Nat_reflTrue; +x_64 = l_Lean_mkApp4(x_62, x_58, x_60, x_61, x_63); +lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -lean_inc(x_2); -lean_inc(x_63); -x_74 = l_Lean_Meta_mkEq(x_1, x_63, x_2, x_3, x_4, x_5, x_68); -if (lean_obj_tag(x_74) == 0) +lean_inc(x_54); +x_65 = l_Lean_Meta_mkEq(x_10, x_54, x_3, x_4, x_5, x_6, x_59); +if (lean_obj_tag(x_65) == 0) { -lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_75 = lean_ctor_get(x_74, 0); +lean_object* x_66; lean_object* x_67; lean_object* x_68; +x_66 = lean_ctor_get(x_65, 0); +lean_inc(x_66); +x_67 = lean_ctor_get(x_65, 1); +lean_inc(x_67); +lean_dec(x_65); +x_68 = l_Lean_Meta_mkExpectedTypeHint(x_64, x_66, x_3, x_4, x_5, x_6, x_67); +if (lean_obj_tag(x_68) == 0) +{ +lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; +x_69 = lean_ctor_get(x_68, 0); +lean_inc(x_69); +x_70 = lean_ctor_get(x_68, 1); +lean_inc(x_70); +if (lean_is_exclusive(x_68)) { + lean_ctor_release(x_68, 0); + lean_ctor_release(x_68, 1); + x_71 = x_68; +} else { + lean_dec_ref(x_68); + x_71 = lean_box(0); +} +lean_ctor_set(x_8, 1, x_69); +lean_ctor_set(x_8, 0, x_54); +x_72 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_72, 0, x_8); +if (lean_is_scalar(x_71)) { + x_73 = lean_alloc_ctor(0, 2, 0); +} else { + x_73 = x_71; +} +lean_ctor_set(x_73, 0, x_72); +lean_ctor_set(x_73, 1, x_70); +return x_73; +} +else +{ +lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; +lean_dec(x_54); +lean_free_object(x_8); +x_74 = lean_ctor_get(x_68, 0); +lean_inc(x_74); +x_75 = lean_ctor_get(x_68, 1); lean_inc(x_75); -x_76 = lean_ctor_get(x_74, 1); -lean_inc(x_76); -lean_dec(x_74); -x_77 = l_Lean_Meta_mkExpectedTypeHint(x_73, x_75, x_2, x_3, x_4, x_5, x_76); -if (lean_obj_tag(x_77) == 0) +if (lean_is_exclusive(x_68)) { + lean_ctor_release(x_68, 0); + lean_ctor_release(x_68, 1); + x_76 = x_68; +} else { + lean_dec_ref(x_68); + x_76 = lean_box(0); +} +if (lean_is_scalar(x_76)) { + x_77 = lean_alloc_ctor(1, 2, 0); +} else { + x_77 = x_76; +} +lean_ctor_set(x_77, 0, x_74); +lean_ctor_set(x_77, 1, x_75); +return x_77; +} +} +else { lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; -x_78 = lean_ctor_get(x_77, 0); +lean_dec(x_64); +lean_dec(x_54); +lean_free_object(x_8); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_78 = lean_ctor_get(x_65, 0); lean_inc(x_78); -x_79 = lean_ctor_get(x_77, 1); +x_79 = lean_ctor_get(x_65, 1); lean_inc(x_79); -if (lean_is_exclusive(x_77)) { - lean_ctor_release(x_77, 0); - lean_ctor_release(x_77, 1); - x_80 = x_77; +if (lean_is_exclusive(x_65)) { + lean_ctor_release(x_65, 0); + lean_ctor_release(x_65, 1); + x_80 = x_65; } else { - lean_dec_ref(x_77); + lean_dec_ref(x_65); x_80 = lean_box(0); } -lean_ctor_set(x_9, 1, x_78); -lean_ctor_set(x_9, 0, x_63); -lean_ctor_set(x_10, 0, x_9); if (lean_is_scalar(x_80)) { - x_81 = lean_alloc_ctor(0, 2, 0); + x_81 = lean_alloc_ctor(1, 2, 0); } else { x_81 = x_80; } -lean_ctor_set(x_81, 0, x_10); +lean_ctor_set(x_81, 0, x_78); lean_ctor_set(x_81, 1, x_79); return x_81; } +} else { lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; -lean_dec(x_63); -lean_free_object(x_10); -lean_free_object(x_9); -x_82 = lean_ctor_get(x_77, 0); +lean_dec(x_54); +lean_dec(x_16); +lean_free_object(x_8); +lean_dec(x_10); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_82 = lean_ctor_get(x_57, 0); lean_inc(x_82); -x_83 = lean_ctor_get(x_77, 1); +x_83 = lean_ctor_get(x_57, 1); lean_inc(x_83); -if (lean_is_exclusive(x_77)) { - lean_ctor_release(x_77, 0); - lean_ctor_release(x_77, 1); - x_84 = x_77; +if (lean_is_exclusive(x_57)) { + lean_ctor_release(x_57, 0); + lean_ctor_release(x_57, 1); + x_84 = x_57; } else { - lean_dec_ref(x_77); + lean_dec_ref(x_57); x_84 = lean_box(0); } if (lean_is_scalar(x_84)) { @@ -648,992 +1545,942 @@ return x_85; } else { -lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; -lean_dec(x_73); -lean_dec(x_63); -lean_free_object(x_10); -lean_free_object(x_9); +lean_object* x_86; lean_object* x_87; +lean_dec(x_54); +lean_dec(x_16); +lean_free_object(x_8); +lean_dec(x_10); +lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_86 = lean_ctor_get(x_74, 0); -lean_inc(x_86); -x_87 = lean_ctor_get(x_74, 1); -lean_inc(x_87); -if (lean_is_exclusive(x_74)) { - lean_ctor_release(x_74, 0); - lean_ctor_release(x_74, 1); - x_88 = x_74; -} else { - lean_dec_ref(x_74); - x_88 = lean_box(0); +lean_dec(x_1); +x_86 = lean_box(0); +x_87 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_87, 0, x_86); +lean_ctor_set(x_87, 1, x_55); +return x_87; } -if (lean_is_scalar(x_88)) { - x_89 = lean_alloc_ctor(1, 2, 0); -} else { - x_89 = x_88; } -lean_ctor_set(x_89, 0, x_86); -lean_ctor_set(x_89, 1, x_87); -return x_89; +} +else +{ +lean_object* x_88; +lean_dec(x_13); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_88 = l_Lean_Meta_Linear_Nat_toContextExpr(x_2, x_3, x_4, x_5, x_6, x_11); +if (lean_obj_tag(x_88) == 0) +{ +lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; +x_89 = lean_ctor_get(x_88, 0); +lean_inc(x_89); +x_90 = lean_ctor_get(x_88, 1); +lean_inc(x_90); +lean_dec(x_88); +x_91 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_1); +x_92 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__11; +x_93 = l_Lean_Meta_Linear_Nat_reflTrue; +x_94 = l_Lean_mkApp3(x_92, x_89, x_91, x_93); +x_95 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__8; +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_96 = l_Lean_Meta_mkEq(x_10, x_95, x_3, x_4, x_5, x_6, x_90); +if (lean_obj_tag(x_96) == 0) +{ +lean_object* x_97; lean_object* x_98; lean_object* x_99; +x_97 = lean_ctor_get(x_96, 0); +lean_inc(x_97); +x_98 = lean_ctor_get(x_96, 1); +lean_inc(x_98); +lean_dec(x_96); +x_99 = l_Lean_Meta_mkExpectedTypeHint(x_94, x_97, x_3, x_4, x_5, x_6, x_98); +if (lean_obj_tag(x_99) == 0) +{ +uint8_t x_100; +x_100 = !lean_is_exclusive(x_99); +if (x_100 == 0) +{ +lean_object* x_101; lean_object* x_102; +x_101 = lean_ctor_get(x_99, 0); +lean_ctor_set(x_8, 1, x_101); +lean_ctor_set(x_8, 0, x_95); +x_102 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_102, 0, x_8); +lean_ctor_set(x_99, 0, x_102); +return x_99; +} +else +{ +lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; +x_103 = lean_ctor_get(x_99, 0); +x_104 = lean_ctor_get(x_99, 1); +lean_inc(x_104); +lean_inc(x_103); +lean_dec(x_99); +lean_ctor_set(x_8, 1, x_103); +lean_ctor_set(x_8, 0, x_95); +x_105 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_105, 0, x_8); +x_106 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_106, 0, x_105); +lean_ctor_set(x_106, 1, x_104); +return x_106; } } else { -lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; -lean_dec(x_63); -lean_dec(x_27); -lean_free_object(x_10); -lean_dec(x_22); -lean_free_object(x_9); +uint8_t x_107; +lean_free_object(x_8); +x_107 = !lean_is_exclusive(x_99); +if (x_107 == 0) +{ +return x_99; +} +else +{ +lean_object* x_108; lean_object* x_109; lean_object* x_110; +x_108 = lean_ctor_get(x_99, 0); +x_109 = lean_ctor_get(x_99, 1); +lean_inc(x_109); +lean_inc(x_108); +lean_dec(x_99); +x_110 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_110, 0, x_108); +lean_ctor_set(x_110, 1, x_109); +return x_110; +} +} +} +else +{ +uint8_t x_111; +lean_dec(x_94); +lean_free_object(x_8); +lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_90 = lean_ctor_get(x_66, 0); -lean_inc(x_90); -x_91 = lean_ctor_get(x_66, 1); -lean_inc(x_91); -if (lean_is_exclusive(x_66)) { - lean_ctor_release(x_66, 0); - lean_ctor_release(x_66, 1); - x_92 = x_66; -} else { - lean_dec_ref(x_66); - x_92 = lean_box(0); +x_111 = !lean_is_exclusive(x_96); +if (x_111 == 0) +{ +return x_96; } -if (lean_is_scalar(x_92)) { - x_93 = lean_alloc_ctor(1, 2, 0); -} else { - x_93 = x_92; +else +{ +lean_object* x_112; lean_object* x_113; lean_object* x_114; +x_112 = lean_ctor_get(x_96, 0); +x_113 = lean_ctor_get(x_96, 1); +lean_inc(x_113); +lean_inc(x_112); +lean_dec(x_96); +x_114 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_114, 0, x_112); +lean_ctor_set(x_114, 1, x_113); +return x_114; } -lean_ctor_set(x_93, 0, x_90); -lean_ctor_set(x_93, 1, x_91); -return x_93; } } else { -lean_object* x_94; lean_object* x_95; -lean_dec(x_63); -lean_dec(x_27); -lean_free_object(x_10); -lean_dec(x_22); -lean_free_object(x_9); -lean_dec(x_19); +uint8_t x_115; +lean_free_object(x_8); +lean_dec(x_10); +lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); lean_dec(x_1); -x_94 = lean_box(0); -x_95 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_95, 0, x_94); -lean_ctor_set(x_95, 1, x_64); -return x_95; +x_115 = !lean_is_exclusive(x_88); +if (x_115 == 0) +{ +return x_88; +} +else +{ +lean_object* x_116; lean_object* x_117; lean_object* x_118; +x_116 = lean_ctor_get(x_88, 0); +x_117 = lean_ctor_get(x_88, 1); +lean_inc(x_117); +lean_inc(x_116); +lean_dec(x_88); +x_118 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_118, 0, x_116); +lean_ctor_set(x_118, 1, x_117); +return x_118; +} } } } else { -lean_object* x_96; -lean_dec(x_24); -lean_dec(x_1); -x_96 = l_Lean_Meta_Linear_Nat_toContextExpr(x_19, x_2, x_3, x_4, x_5, x_17); -if (lean_obj_tag(x_96) == 0) -{ -uint8_t x_97; -x_97 = !lean_is_exclusive(x_96); -if (x_97 == 0) -{ -lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; -x_98 = lean_ctor_get(x_96, 0); -x_99 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_22); -x_100 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__9; -x_101 = l_Lean_Meta_Linear_Nat_reflTrue; -x_102 = l_Lean_mkApp3(x_100, x_98, x_99, x_101); -x_103 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__12; -lean_ctor_set(x_9, 1, x_102); -lean_ctor_set(x_9, 0, x_103); -lean_ctor_set(x_10, 0, x_9); -lean_ctor_set(x_96, 0, x_10); -return x_96; +lean_object* x_119; +lean_dec(x_13); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_119 = l_Lean_Meta_Linear_Nat_toContextExpr(x_2, x_3, x_4, x_5, x_6, x_11); +if (lean_obj_tag(x_119) == 0) +{ +lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; +x_120 = lean_ctor_get(x_119, 0); +lean_inc(x_120); +x_121 = lean_ctor_get(x_119, 1); +lean_inc(x_121); +lean_dec(x_119); +x_122 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_1); +x_123 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__17; +x_124 = l_Lean_Meta_Linear_Nat_reflTrue; +x_125 = l_Lean_mkApp3(x_123, x_120, x_122, x_124); +x_126 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__14; +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_127 = l_Lean_Meta_mkEq(x_10, x_126, x_3, x_4, x_5, x_6, x_121); +if (lean_obj_tag(x_127) == 0) +{ +lean_object* x_128; lean_object* x_129; lean_object* x_130; +x_128 = lean_ctor_get(x_127, 0); +lean_inc(x_128); +x_129 = lean_ctor_get(x_127, 1); +lean_inc(x_129); +lean_dec(x_127); +x_130 = l_Lean_Meta_mkExpectedTypeHint(x_125, x_128, x_3, x_4, x_5, x_6, x_129); +if (lean_obj_tag(x_130) == 0) +{ +uint8_t x_131; +x_131 = !lean_is_exclusive(x_130); +if (x_131 == 0) +{ +lean_object* x_132; lean_object* x_133; +x_132 = lean_ctor_get(x_130, 0); +lean_ctor_set(x_8, 1, x_132); +lean_ctor_set(x_8, 0, x_126); +x_133 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_133, 0, x_8); +lean_ctor_set(x_130, 0, x_133); +return x_130; } else { -lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; -x_104 = lean_ctor_get(x_96, 0); -x_105 = lean_ctor_get(x_96, 1); -lean_inc(x_105); -lean_inc(x_104); -lean_dec(x_96); -x_106 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_22); -x_107 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__9; -x_108 = l_Lean_Meta_Linear_Nat_reflTrue; -x_109 = l_Lean_mkApp3(x_107, x_104, x_106, x_108); -x_110 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__12; -lean_ctor_set(x_9, 1, x_109); -lean_ctor_set(x_9, 0, x_110); -lean_ctor_set(x_10, 0, x_9); -x_111 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_111, 0, x_10); -lean_ctor_set(x_111, 1, x_105); -return x_111; +lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; +x_134 = lean_ctor_get(x_130, 0); +x_135 = lean_ctor_get(x_130, 1); +lean_inc(x_135); +lean_inc(x_134); +lean_dec(x_130); +lean_ctor_set(x_8, 1, x_134); +lean_ctor_set(x_8, 0, x_126); +x_136 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_136, 0, x_8); +x_137 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_137, 0, x_136); +lean_ctor_set(x_137, 1, x_135); +return x_137; } } else { -uint8_t x_112; -lean_free_object(x_10); -lean_dec(x_22); -lean_free_object(x_9); -x_112 = !lean_is_exclusive(x_96); -if (x_112 == 0) +uint8_t x_138; +lean_free_object(x_8); +x_138 = !lean_is_exclusive(x_130); +if (x_138 == 0) { -return x_96; +return x_130; } else { -lean_object* x_113; lean_object* x_114; lean_object* x_115; -x_113 = lean_ctor_get(x_96, 0); -x_114 = lean_ctor_get(x_96, 1); -lean_inc(x_114); -lean_inc(x_113); -lean_dec(x_96); -x_115 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_115, 0, x_113); -lean_ctor_set(x_115, 1, x_114); -return x_115; -} +lean_object* x_139; lean_object* x_140; lean_object* x_141; +x_139 = lean_ctor_get(x_130, 0); +x_140 = lean_ctor_get(x_130, 1); +lean_inc(x_140); +lean_inc(x_139); +lean_dec(x_130); +x_141 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_141, 0, x_139); +lean_ctor_set(x_141, 1, x_140); +return x_141; } } } else { -lean_object* x_116; -lean_dec(x_24); -lean_dec(x_1); -x_116 = l_Lean_Meta_Linear_Nat_toContextExpr(x_19, x_2, x_3, x_4, x_5, x_17); -if (lean_obj_tag(x_116) == 0) -{ -uint8_t x_117; -x_117 = !lean_is_exclusive(x_116); -if (x_117 == 0) +uint8_t x_142; +lean_dec(x_125); +lean_free_object(x_8); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_142 = !lean_is_exclusive(x_127); +if (x_142 == 0) { -lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; -x_118 = lean_ctor_get(x_116, 0); -x_119 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_22); -x_120 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__15; -x_121 = l_Lean_Meta_Linear_Nat_reflTrue; -x_122 = l_Lean_mkApp3(x_120, x_118, x_119, x_121); -x_123 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__18; -lean_ctor_set(x_9, 1, x_122); -lean_ctor_set(x_9, 0, x_123); -lean_ctor_set(x_10, 0, x_9); -lean_ctor_set(x_116, 0, x_10); -return x_116; +return x_127; } else { -lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; -x_124 = lean_ctor_get(x_116, 0); -x_125 = lean_ctor_get(x_116, 1); -lean_inc(x_125); -lean_inc(x_124); -lean_dec(x_116); -x_126 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_22); -x_127 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__15; -x_128 = l_Lean_Meta_Linear_Nat_reflTrue; -x_129 = l_Lean_mkApp3(x_127, x_124, x_126, x_128); -x_130 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__18; -lean_ctor_set(x_9, 1, x_129); -lean_ctor_set(x_9, 0, x_130); -lean_ctor_set(x_10, 0, x_9); -x_131 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_131, 0, x_10); -lean_ctor_set(x_131, 1, x_125); -return x_131; +lean_object* x_143; lean_object* x_144; lean_object* x_145; +x_143 = lean_ctor_get(x_127, 0); +x_144 = lean_ctor_get(x_127, 1); +lean_inc(x_144); +lean_inc(x_143); +lean_dec(x_127); +x_145 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_145, 0, x_143); +lean_ctor_set(x_145, 1, x_144); +return x_145; +} } } else { -uint8_t x_132; -lean_free_object(x_10); -lean_dec(x_22); -lean_free_object(x_9); -x_132 = !lean_is_exclusive(x_116); -if (x_132 == 0) +uint8_t x_146; +lean_free_object(x_8); +lean_dec(x_10); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_146 = !lean_is_exclusive(x_119); +if (x_146 == 0) { -return x_116; +return x_119; } else { -lean_object* x_133; lean_object* x_134; lean_object* x_135; -x_133 = lean_ctor_get(x_116, 0); -x_134 = lean_ctor_get(x_116, 1); -lean_inc(x_134); -lean_inc(x_133); -lean_dec(x_116); -x_135 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_135, 0, x_133); -lean_ctor_set(x_135, 1, x_134); -return x_135; +lean_object* x_147; lean_object* x_148; lean_object* x_149; +x_147 = lean_ctor_get(x_119, 0); +x_148 = lean_ctor_get(x_119, 1); +lean_inc(x_148); +lean_inc(x_147); +lean_dec(x_119); +x_149 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_149, 0, x_147); +lean_ctor_set(x_149, 1, x_148); +return x_149; } } } } else { -lean_object* x_136; lean_object* x_137; lean_object* x_138; uint8_t x_139; -x_136 = lean_ctor_get(x_10, 0); -lean_inc(x_136); -lean_dec(x_10); -lean_inc(x_136); -x_137 = l_Nat_Linear_ExprCnstr_toPoly(x_136); -x_138 = l_Nat_Linear_PolyCnstr_norm(x_137); -x_139 = l_Nat_Linear_PolyCnstr_isUnsat(x_138); -if (x_139 == 0) -{ -uint8_t x_140; -x_140 = l_Nat_Linear_PolyCnstr_isValid(x_138); -if (x_140 == 0) -{ -lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; uint8_t x_146; -x_141 = l_Nat_Linear_PolyCnstr_toExpr(x_138); -lean_inc(x_141); -x_142 = l_Lean_Meta_Linear_Nat_LinearCnstr_toArith(x_19, x_141, x_2, x_3, x_4, x_5, x_17); -x_143 = lean_ctor_get(x_142, 0); -lean_inc(x_143); -x_144 = lean_ctor_get(x_142, 1); -lean_inc(x_144); -if (lean_is_exclusive(x_142)) { - lean_ctor_release(x_142, 0); - lean_ctor_release(x_142, 1); - x_145 = x_142; +lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; uint8_t x_154; +x_150 = lean_ctor_get(x_8, 0); +x_151 = lean_ctor_get(x_8, 1); +lean_inc(x_151); +lean_inc(x_150); +lean_dec(x_8); +lean_inc(x_1); +x_152 = l_Nat_Linear_ExprCnstr_toPoly(x_1); +x_153 = l_Nat_Linear_PolyCnstr_norm(x_152); +x_154 = l_Nat_Linear_PolyCnstr_isUnsat(x_153); +if (x_154 == 0) +{ +uint8_t x_155; +x_155 = l_Nat_Linear_PolyCnstr_isValid(x_153); +if (x_155 == 0) +{ +lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; uint8_t x_161; +x_156 = l_Nat_Linear_PolyCnstr_toExpr(x_153); +lean_inc(x_156); +x_157 = l_Lean_Meta_Linear_Nat_LinearCnstr_toArith(x_2, x_156, x_3, x_4, x_5, x_6, x_151); +x_158 = lean_ctor_get(x_157, 0); +lean_inc(x_158); +x_159 = lean_ctor_get(x_157, 1); +lean_inc(x_159); +if (lean_is_exclusive(x_157)) { + lean_ctor_release(x_157, 0); + lean_ctor_release(x_157, 1); + x_160 = x_157; } else { - lean_dec_ref(x_142); - x_145 = lean_box(0); + lean_dec_ref(x_157); + x_160 = lean_box(0); } -x_146 = lean_expr_eqv(x_143, x_1); -if (x_146 == 0) +x_161 = lean_expr_eqv(x_158, x_150); +if (x_161 == 0) { -lean_object* x_147; -lean_dec(x_145); +lean_object* x_162; +lean_dec(x_160); +lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -lean_inc(x_2); -x_147 = l_Lean_Meta_Linear_Nat_toContextExpr(x_19, x_2, x_3, x_4, x_5, x_144); -if (lean_obj_tag(x_147) == 0) +x_162 = l_Lean_Meta_Linear_Nat_toContextExpr(x_2, x_3, x_4, x_5, x_6, x_159); +if (lean_obj_tag(x_162) == 0) { -lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; -x_148 = lean_ctor_get(x_147, 0); -lean_inc(x_148); -x_149 = lean_ctor_get(x_147, 1); -lean_inc(x_149); -lean_dec(x_147); -x_150 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_136); -x_151 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_141); -x_152 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__6; -x_153 = l_Lean_Meta_Linear_Nat_reflTrue; -x_154 = l_Lean_mkApp4(x_152, x_148, x_150, x_151, x_153); +lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; +x_163 = lean_ctor_get(x_162, 0); +lean_inc(x_163); +x_164 = lean_ctor_get(x_162, 1); +lean_inc(x_164); +lean_dec(x_162); +x_165 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_1); +x_166 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_156); +x_167 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__5; +x_168 = l_Lean_Meta_Linear_Nat_reflTrue; +x_169 = l_Lean_mkApp4(x_167, x_163, x_165, x_166, x_168); +lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -lean_inc(x_2); -lean_inc(x_143); -x_155 = l_Lean_Meta_mkEq(x_1, x_143, x_2, x_3, x_4, x_5, x_149); -if (lean_obj_tag(x_155) == 0) -{ -lean_object* x_156; lean_object* x_157; lean_object* x_158; -x_156 = lean_ctor_get(x_155, 0); -lean_inc(x_156); -x_157 = lean_ctor_get(x_155, 1); -lean_inc(x_157); -lean_dec(x_155); -x_158 = l_Lean_Meta_mkExpectedTypeHint(x_154, x_156, x_2, x_3, x_4, x_5, x_157); -if (lean_obj_tag(x_158) == 0) -{ -lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; -x_159 = lean_ctor_get(x_158, 0); -lean_inc(x_159); -x_160 = lean_ctor_get(x_158, 1); -lean_inc(x_160); -if (lean_is_exclusive(x_158)) { - lean_ctor_release(x_158, 0); - lean_ctor_release(x_158, 1); - x_161 = x_158; +lean_inc(x_158); +x_170 = l_Lean_Meta_mkEq(x_150, x_158, x_3, x_4, x_5, x_6, x_164); +if (lean_obj_tag(x_170) == 0) +{ +lean_object* x_171; lean_object* x_172; lean_object* x_173; +x_171 = lean_ctor_get(x_170, 0); +lean_inc(x_171); +x_172 = lean_ctor_get(x_170, 1); +lean_inc(x_172); +lean_dec(x_170); +x_173 = l_Lean_Meta_mkExpectedTypeHint(x_169, x_171, x_3, x_4, x_5, x_6, x_172); +if (lean_obj_tag(x_173) == 0) +{ +lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; +x_174 = lean_ctor_get(x_173, 0); +lean_inc(x_174); +x_175 = lean_ctor_get(x_173, 1); +lean_inc(x_175); +if (lean_is_exclusive(x_173)) { + lean_ctor_release(x_173, 0); + lean_ctor_release(x_173, 1); + x_176 = x_173; } else { - lean_dec_ref(x_158); - x_161 = lean_box(0); -} -lean_ctor_set(x_9, 1, x_159); -lean_ctor_set(x_9, 0, x_143); -x_162 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_162, 0, x_9); -if (lean_is_scalar(x_161)) { - x_163 = lean_alloc_ctor(0, 2, 0); + lean_dec_ref(x_173); + x_176 = lean_box(0); +} +x_177 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_177, 0, x_158); +lean_ctor_set(x_177, 1, x_174); +x_178 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_178, 0, x_177); +if (lean_is_scalar(x_176)) { + x_179 = lean_alloc_ctor(0, 2, 0); } else { - x_163 = x_161; + x_179 = x_176; } -lean_ctor_set(x_163, 0, x_162); -lean_ctor_set(x_163, 1, x_160); -return x_163; +lean_ctor_set(x_179, 0, x_178); +lean_ctor_set(x_179, 1, x_175); +return x_179; } else { -lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; -lean_dec(x_143); -lean_free_object(x_9); -x_164 = lean_ctor_get(x_158, 0); -lean_inc(x_164); -x_165 = lean_ctor_get(x_158, 1); -lean_inc(x_165); -if (lean_is_exclusive(x_158)) { - lean_ctor_release(x_158, 0); - lean_ctor_release(x_158, 1); - x_166 = x_158; +lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; +lean_dec(x_158); +x_180 = lean_ctor_get(x_173, 0); +lean_inc(x_180); +x_181 = lean_ctor_get(x_173, 1); +lean_inc(x_181); +if (lean_is_exclusive(x_173)) { + lean_ctor_release(x_173, 0); + lean_ctor_release(x_173, 1); + x_182 = x_173; } else { - lean_dec_ref(x_158); - x_166 = lean_box(0); + lean_dec_ref(x_173); + x_182 = lean_box(0); } -if (lean_is_scalar(x_166)) { - x_167 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_182)) { + x_183 = lean_alloc_ctor(1, 2, 0); } else { - x_167 = x_166; + x_183 = x_182; } -lean_ctor_set(x_167, 0, x_164); -lean_ctor_set(x_167, 1, x_165); -return x_167; +lean_ctor_set(x_183, 0, x_180); +lean_ctor_set(x_183, 1, x_181); +return x_183; } } else { -lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; -lean_dec(x_154); -lean_dec(x_143); -lean_free_object(x_9); +lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; +lean_dec(x_169); +lean_dec(x_158); +lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); -x_168 = lean_ctor_get(x_155, 0); -lean_inc(x_168); -x_169 = lean_ctor_get(x_155, 1); -lean_inc(x_169); -if (lean_is_exclusive(x_155)) { - lean_ctor_release(x_155, 0); - lean_ctor_release(x_155, 1); - x_170 = x_155; +x_184 = lean_ctor_get(x_170, 0); +lean_inc(x_184); +x_185 = lean_ctor_get(x_170, 1); +lean_inc(x_185); +if (lean_is_exclusive(x_170)) { + lean_ctor_release(x_170, 0); + lean_ctor_release(x_170, 1); + x_186 = x_170; } else { - lean_dec_ref(x_155); - x_170 = lean_box(0); + lean_dec_ref(x_170); + x_186 = lean_box(0); } -if (lean_is_scalar(x_170)) { - x_171 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_186)) { + x_187 = lean_alloc_ctor(1, 2, 0); } else { - x_171 = x_170; + x_187 = x_186; } -lean_ctor_set(x_171, 0, x_168); -lean_ctor_set(x_171, 1, x_169); -return x_171; +lean_ctor_set(x_187, 0, x_184); +lean_ctor_set(x_187, 1, x_185); +return x_187; } } else { -lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; -lean_dec(x_143); -lean_dec(x_141); -lean_dec(x_136); -lean_free_object(x_9); +lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; +lean_dec(x_158); +lean_dec(x_156); +lean_dec(x_150); +lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); lean_dec(x_1); -x_172 = lean_ctor_get(x_147, 0); -lean_inc(x_172); -x_173 = lean_ctor_get(x_147, 1); -lean_inc(x_173); -if (lean_is_exclusive(x_147)) { - lean_ctor_release(x_147, 0); - lean_ctor_release(x_147, 1); - x_174 = x_147; +x_188 = lean_ctor_get(x_162, 0); +lean_inc(x_188); +x_189 = lean_ctor_get(x_162, 1); +lean_inc(x_189); +if (lean_is_exclusive(x_162)) { + lean_ctor_release(x_162, 0); + lean_ctor_release(x_162, 1); + x_190 = x_162; } else { - lean_dec_ref(x_147); - x_174 = lean_box(0); + lean_dec_ref(x_162); + x_190 = lean_box(0); } -if (lean_is_scalar(x_174)) { - x_175 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_190)) { + x_191 = lean_alloc_ctor(1, 2, 0); } else { - x_175 = x_174; + x_191 = x_190; } -lean_ctor_set(x_175, 0, x_172); -lean_ctor_set(x_175, 1, x_173); -return x_175; +lean_ctor_set(x_191, 0, x_188); +lean_ctor_set(x_191, 1, x_189); +return x_191; } } else { -lean_object* x_176; lean_object* x_177; -lean_dec(x_143); -lean_dec(x_141); -lean_dec(x_136); -lean_free_object(x_9); -lean_dec(x_19); +lean_object* x_192; lean_object* x_193; +lean_dec(x_158); +lean_dec(x_156); +lean_dec(x_150); +lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_176 = lean_box(0); -if (lean_is_scalar(x_145)) { - x_177 = lean_alloc_ctor(0, 2, 0); +x_192 = lean_box(0); +if (lean_is_scalar(x_160)) { + x_193 = lean_alloc_ctor(0, 2, 0); } else { - x_177 = x_145; + x_193 = x_160; } -lean_ctor_set(x_177, 0, x_176); -lean_ctor_set(x_177, 1, x_144); -return x_177; +lean_ctor_set(x_193, 0, x_192); +lean_ctor_set(x_193, 1, x_159); +return x_193; } } else { -lean_object* x_178; -lean_dec(x_138); -lean_dec(x_1); -x_178 = l_Lean_Meta_Linear_Nat_toContextExpr(x_19, x_2, x_3, x_4, x_5, x_17); -if (lean_obj_tag(x_178) == 0) +lean_object* x_194; +lean_dec(x_153); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_194 = l_Lean_Meta_Linear_Nat_toContextExpr(x_2, x_3, x_4, x_5, x_6, x_151); +if (lean_obj_tag(x_194) == 0) { -lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; -x_179 = lean_ctor_get(x_178, 0); -lean_inc(x_179); -x_180 = lean_ctor_get(x_178, 1); -lean_inc(x_180); -if (lean_is_exclusive(x_178)) { - lean_ctor_release(x_178, 0); - lean_ctor_release(x_178, 1); - x_181 = x_178; -} else { - lean_dec_ref(x_178); - x_181 = lean_box(0); -} -x_182 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_136); -x_183 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__9; -x_184 = l_Lean_Meta_Linear_Nat_reflTrue; -x_185 = l_Lean_mkApp3(x_183, x_179, x_182, x_184); -x_186 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__12; -lean_ctor_set(x_9, 1, x_185); -lean_ctor_set(x_9, 0, x_186); -x_187 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_187, 0, x_9); -if (lean_is_scalar(x_181)) { - x_188 = lean_alloc_ctor(0, 2, 0); -} else { - x_188 = x_181; -} -lean_ctor_set(x_188, 0, x_187); -lean_ctor_set(x_188, 1, x_180); -return x_188; -} -else -{ -lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; -lean_dec(x_136); -lean_free_object(x_9); -x_189 = lean_ctor_get(x_178, 0); -lean_inc(x_189); -x_190 = lean_ctor_get(x_178, 1); -lean_inc(x_190); -if (lean_is_exclusive(x_178)) { - lean_ctor_release(x_178, 0); - lean_ctor_release(x_178, 1); - x_191 = x_178; +lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; +x_195 = lean_ctor_get(x_194, 0); +lean_inc(x_195); +x_196 = lean_ctor_get(x_194, 1); +lean_inc(x_196); +lean_dec(x_194); +x_197 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_1); +x_198 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__11; +x_199 = l_Lean_Meta_Linear_Nat_reflTrue; +x_200 = l_Lean_mkApp3(x_198, x_195, x_197, x_199); +x_201 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__8; +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_202 = l_Lean_Meta_mkEq(x_150, x_201, x_3, x_4, x_5, x_6, x_196); +if (lean_obj_tag(x_202) == 0) +{ +lean_object* x_203; lean_object* x_204; lean_object* x_205; +x_203 = lean_ctor_get(x_202, 0); +lean_inc(x_203); +x_204 = lean_ctor_get(x_202, 1); +lean_inc(x_204); +lean_dec(x_202); +x_205 = l_Lean_Meta_mkExpectedTypeHint(x_200, x_203, x_3, x_4, x_5, x_6, x_204); +if (lean_obj_tag(x_205) == 0) +{ +lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; +x_206 = lean_ctor_get(x_205, 0); +lean_inc(x_206); +x_207 = lean_ctor_get(x_205, 1); +lean_inc(x_207); +if (lean_is_exclusive(x_205)) { + lean_ctor_release(x_205, 0); + lean_ctor_release(x_205, 1); + x_208 = x_205; +} else { + lean_dec_ref(x_205); + x_208 = lean_box(0); +} +x_209 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_209, 0, x_201); +lean_ctor_set(x_209, 1, x_206); +x_210 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_210, 0, x_209); +if (lean_is_scalar(x_208)) { + x_211 = lean_alloc_ctor(0, 2, 0); } else { - lean_dec_ref(x_178); - x_191 = lean_box(0); + x_211 = x_208; } -if (lean_is_scalar(x_191)) { - x_192 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_211, 0, x_210); +lean_ctor_set(x_211, 1, x_207); +return x_211; +} +else +{ +lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; +x_212 = lean_ctor_get(x_205, 0); +lean_inc(x_212); +x_213 = lean_ctor_get(x_205, 1); +lean_inc(x_213); +if (lean_is_exclusive(x_205)) { + lean_ctor_release(x_205, 0); + lean_ctor_release(x_205, 1); + x_214 = x_205; } else { - x_192 = x_191; + lean_dec_ref(x_205); + x_214 = lean_box(0); } -lean_ctor_set(x_192, 0, x_189); -lean_ctor_set(x_192, 1, x_190); -return x_192; +if (lean_is_scalar(x_214)) { + x_215 = lean_alloc_ctor(1, 2, 0); +} else { + x_215 = x_214; } +lean_ctor_set(x_215, 0, x_212); +lean_ctor_set(x_215, 1, x_213); +return x_215; } } else { -lean_object* x_193; -lean_dec(x_138); -lean_dec(x_1); -x_193 = l_Lean_Meta_Linear_Nat_toContextExpr(x_19, x_2, x_3, x_4, x_5, x_17); -if (lean_obj_tag(x_193) == 0) -{ -lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; -x_194 = lean_ctor_get(x_193, 0); -lean_inc(x_194); -x_195 = lean_ctor_get(x_193, 1); -lean_inc(x_195); -if (lean_is_exclusive(x_193)) { - lean_ctor_release(x_193, 0); - lean_ctor_release(x_193, 1); - x_196 = x_193; +lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; +lean_dec(x_200); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_216 = lean_ctor_get(x_202, 0); +lean_inc(x_216); +x_217 = lean_ctor_get(x_202, 1); +lean_inc(x_217); +if (lean_is_exclusive(x_202)) { + lean_ctor_release(x_202, 0); + lean_ctor_release(x_202, 1); + x_218 = x_202; } else { - lean_dec_ref(x_193); - x_196 = lean_box(0); + lean_dec_ref(x_202); + x_218 = lean_box(0); } -x_197 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_136); -x_198 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__15; -x_199 = l_Lean_Meta_Linear_Nat_reflTrue; -x_200 = l_Lean_mkApp3(x_198, x_194, x_197, x_199); -x_201 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__18; -lean_ctor_set(x_9, 1, x_200); -lean_ctor_set(x_9, 0, x_201); -x_202 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_202, 0, x_9); -if (lean_is_scalar(x_196)) { - x_203 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_218)) { + x_219 = lean_alloc_ctor(1, 2, 0); } else { - x_203 = x_196; + x_219 = x_218; +} +lean_ctor_set(x_219, 0, x_216); +lean_ctor_set(x_219, 1, x_217); +return x_219; } -lean_ctor_set(x_203, 0, x_202); -lean_ctor_set(x_203, 1, x_195); -return x_203; } else { -lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; -lean_dec(x_136); -lean_free_object(x_9); -x_204 = lean_ctor_get(x_193, 0); -lean_inc(x_204); -x_205 = lean_ctor_get(x_193, 1); -lean_inc(x_205); -if (lean_is_exclusive(x_193)) { - lean_ctor_release(x_193, 0); - lean_ctor_release(x_193, 1); - x_206 = x_193; +lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; +lean_dec(x_150); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_220 = lean_ctor_get(x_194, 0); +lean_inc(x_220); +x_221 = lean_ctor_get(x_194, 1); +lean_inc(x_221); +if (lean_is_exclusive(x_194)) { + lean_ctor_release(x_194, 0); + lean_ctor_release(x_194, 1); + x_222 = x_194; } else { - lean_dec_ref(x_193); - x_206 = lean_box(0); + lean_dec_ref(x_194); + x_222 = lean_box(0); } -if (lean_is_scalar(x_206)) { - x_207 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_222)) { + x_223 = lean_alloc_ctor(1, 2, 0); } else { - x_207 = x_206; -} -lean_ctor_set(x_207, 0, x_204); -lean_ctor_set(x_207, 1, x_205); -return x_207; + x_223 = x_222; } +lean_ctor_set(x_223, 0, x_220); +lean_ctor_set(x_223, 1, x_221); +return x_223; } } } else { -lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; uint8_t x_213; -x_208 = lean_ctor_get(x_9, 1); -lean_inc(x_208); -lean_dec(x_9); -x_209 = lean_ctor_get(x_10, 0); -lean_inc(x_209); -if (lean_is_exclusive(x_10)) { - lean_ctor_release(x_10, 0); - x_210 = x_10; -} else { - lean_dec_ref(x_10); - x_210 = lean_box(0); -} -lean_inc(x_209); -x_211 = l_Nat_Linear_ExprCnstr_toPoly(x_209); -x_212 = l_Nat_Linear_PolyCnstr_norm(x_211); -x_213 = l_Nat_Linear_PolyCnstr_isUnsat(x_212); -if (x_213 == 0) -{ -uint8_t x_214; -x_214 = l_Nat_Linear_PolyCnstr_isValid(x_212); -if (x_214 == 0) -{ -lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; uint8_t x_220; -x_215 = l_Nat_Linear_PolyCnstr_toExpr(x_212); -lean_inc(x_215); -x_216 = l_Lean_Meta_Linear_Nat_LinearCnstr_toArith(x_208, x_215, x_2, x_3, x_4, x_5, x_17); -x_217 = lean_ctor_get(x_216, 0); -lean_inc(x_217); -x_218 = lean_ctor_get(x_216, 1); -lean_inc(x_218); -if (lean_is_exclusive(x_216)) { - lean_ctor_release(x_216, 0); - lean_ctor_release(x_216, 1); - x_219 = x_216; -} else { - lean_dec_ref(x_216); - x_219 = lean_box(0); -} -x_220 = lean_expr_eqv(x_217, x_1); -if (x_220 == 0) -{ -lean_object* x_221; -lean_dec(x_219); +lean_object* x_224; +lean_dec(x_153); +lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -lean_inc(x_2); -x_221 = l_Lean_Meta_Linear_Nat_toContextExpr(x_208, x_2, x_3, x_4, x_5, x_218); -if (lean_obj_tag(x_221) == 0) -{ -lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; -x_222 = lean_ctor_get(x_221, 0); -lean_inc(x_222); -x_223 = lean_ctor_get(x_221, 1); -lean_inc(x_223); -lean_dec(x_221); -x_224 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_209); -x_225 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_215); -x_226 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__6; -x_227 = l_Lean_Meta_Linear_Nat_reflTrue; -x_228 = l_Lean_mkApp4(x_226, x_222, x_224, x_225, x_227); +x_224 = l_Lean_Meta_Linear_Nat_toContextExpr(x_2, x_3, x_4, x_5, x_6, x_151); +if (lean_obj_tag(x_224) == 0) +{ +lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; +x_225 = lean_ctor_get(x_224, 0); +lean_inc(x_225); +x_226 = lean_ctor_get(x_224, 1); +lean_inc(x_226); +lean_dec(x_224); +x_227 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_1); +x_228 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__17; +x_229 = l_Lean_Meta_Linear_Nat_reflTrue; +x_230 = l_Lean_mkApp3(x_228, x_225, x_227, x_229); +x_231 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__14; +lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -lean_inc(x_2); -lean_inc(x_217); -x_229 = l_Lean_Meta_mkEq(x_1, x_217, x_2, x_3, x_4, x_5, x_223); -if (lean_obj_tag(x_229) == 0) -{ -lean_object* x_230; lean_object* x_231; lean_object* x_232; -x_230 = lean_ctor_get(x_229, 0); -lean_inc(x_230); -x_231 = lean_ctor_get(x_229, 1); -lean_inc(x_231); -lean_dec(x_229); -x_232 = l_Lean_Meta_mkExpectedTypeHint(x_228, x_230, x_2, x_3, x_4, x_5, x_231); +x_232 = l_Lean_Meta_mkEq(x_150, x_231, x_3, x_4, x_5, x_6, x_226); if (lean_obj_tag(x_232) == 0) { -lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; +lean_object* x_233; lean_object* x_234; lean_object* x_235; x_233 = lean_ctor_get(x_232, 0); lean_inc(x_233); x_234 = lean_ctor_get(x_232, 1); lean_inc(x_234); -if (lean_is_exclusive(x_232)) { - lean_ctor_release(x_232, 0); - lean_ctor_release(x_232, 1); - x_235 = x_232; -} else { - lean_dec_ref(x_232); - x_235 = lean_box(0); -} -x_236 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_236, 0, x_217); -lean_ctor_set(x_236, 1, x_233); -if (lean_is_scalar(x_210)) { - x_237 = lean_alloc_ctor(1, 1, 0); -} else { - x_237 = x_210; -} -lean_ctor_set(x_237, 0, x_236); -if (lean_is_scalar(x_235)) { - x_238 = lean_alloc_ctor(0, 2, 0); -} else { +lean_dec(x_232); +x_235 = l_Lean_Meta_mkExpectedTypeHint(x_230, x_233, x_3, x_4, x_5, x_6, x_234); +if (lean_obj_tag(x_235) == 0) +{ +lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; +x_236 = lean_ctor_get(x_235, 0); +lean_inc(x_236); +x_237 = lean_ctor_get(x_235, 1); +lean_inc(x_237); +if (lean_is_exclusive(x_235)) { + lean_ctor_release(x_235, 0); + lean_ctor_release(x_235, 1); x_238 = x_235; -} -lean_ctor_set(x_238, 0, x_237); -lean_ctor_set(x_238, 1, x_234); -return x_238; -} -else -{ -lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; -lean_dec(x_217); -lean_dec(x_210); -x_239 = lean_ctor_get(x_232, 0); -lean_inc(x_239); -x_240 = lean_ctor_get(x_232, 1); -lean_inc(x_240); -if (lean_is_exclusive(x_232)) { - lean_ctor_release(x_232, 0); - lean_ctor_release(x_232, 1); - x_241 = x_232; } else { - lean_dec_ref(x_232); - x_241 = lean_box(0); -} -if (lean_is_scalar(x_241)) { - x_242 = lean_alloc_ctor(1, 2, 0); + lean_dec_ref(x_235); + x_238 = lean_box(0); +} +x_239 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_239, 0, x_231); +lean_ctor_set(x_239, 1, x_236); +x_240 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_240, 0, x_239); +if (lean_is_scalar(x_238)) { + x_241 = lean_alloc_ctor(0, 2, 0); } else { - x_242 = x_241; -} -lean_ctor_set(x_242, 0, x_239); -lean_ctor_set(x_242, 1, x_240); -return x_242; + x_241 = x_238; } +lean_ctor_set(x_241, 0, x_240); +lean_ctor_set(x_241, 1, x_237); +return x_241; } else { -lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; -lean_dec(x_228); -lean_dec(x_217); -lean_dec(x_210); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_243 = lean_ctor_get(x_229, 0); +lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; +x_242 = lean_ctor_get(x_235, 0); +lean_inc(x_242); +x_243 = lean_ctor_get(x_235, 1); lean_inc(x_243); -x_244 = lean_ctor_get(x_229, 1); -lean_inc(x_244); -if (lean_is_exclusive(x_229)) { - lean_ctor_release(x_229, 0); - lean_ctor_release(x_229, 1); - x_245 = x_229; +if (lean_is_exclusive(x_235)) { + lean_ctor_release(x_235, 0); + lean_ctor_release(x_235, 1); + x_244 = x_235; } else { - lean_dec_ref(x_229); - x_245 = lean_box(0); + lean_dec_ref(x_235); + x_244 = lean_box(0); } -if (lean_is_scalar(x_245)) { - x_246 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_244)) { + x_245 = lean_alloc_ctor(1, 2, 0); } else { - x_246 = x_245; + x_245 = x_244; } -lean_ctor_set(x_246, 0, x_243); -lean_ctor_set(x_246, 1, x_244); -return x_246; +lean_ctor_set(x_245, 0, x_242); +lean_ctor_set(x_245, 1, x_243); +return x_245; } } else { -lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; -lean_dec(x_217); -lean_dec(x_215); -lean_dec(x_210); -lean_dec(x_209); +lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; +lean_dec(x_230); +lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_247 = lean_ctor_get(x_221, 0); +x_246 = lean_ctor_get(x_232, 0); +lean_inc(x_246); +x_247 = lean_ctor_get(x_232, 1); lean_inc(x_247); -x_248 = lean_ctor_get(x_221, 1); -lean_inc(x_248); -if (lean_is_exclusive(x_221)) { - lean_ctor_release(x_221, 0); - lean_ctor_release(x_221, 1); - x_249 = x_221; +if (lean_is_exclusive(x_232)) { + lean_ctor_release(x_232, 0); + lean_ctor_release(x_232, 1); + x_248 = x_232; } else { - lean_dec_ref(x_221); - x_249 = lean_box(0); + lean_dec_ref(x_232); + x_248 = lean_box(0); } -if (lean_is_scalar(x_249)) { - x_250 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_248)) { + x_249 = lean_alloc_ctor(1, 2, 0); } else { - x_250 = x_249; + x_249 = x_248; } -lean_ctor_set(x_250, 0, x_247); -lean_ctor_set(x_250, 1, x_248); -return x_250; +lean_ctor_set(x_249, 0, x_246); +lean_ctor_set(x_249, 1, x_247); +return x_249; } } else { -lean_object* x_251; lean_object* x_252; -lean_dec(x_217); -lean_dec(x_215); -lean_dec(x_210); -lean_dec(x_209); -lean_dec(x_208); +lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; +lean_dec(x_150); +lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_251 = lean_box(0); -if (lean_is_scalar(x_219)) { - x_252 = lean_alloc_ctor(0, 2, 0); -} else { - x_252 = x_219; -} -lean_ctor_set(x_252, 0, x_251); -lean_ctor_set(x_252, 1, x_218); -return x_252; -} -} -else -{ -lean_object* x_253; -lean_dec(x_212); lean_dec(x_1); -x_253 = l_Lean_Meta_Linear_Nat_toContextExpr(x_208, x_2, x_3, x_4, x_5, x_17); -if (lean_obj_tag(x_253) == 0) -{ -lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; -x_254 = lean_ctor_get(x_253, 0); -lean_inc(x_254); -x_255 = lean_ctor_get(x_253, 1); -lean_inc(x_255); -if (lean_is_exclusive(x_253)) { - lean_ctor_release(x_253, 0); - lean_ctor_release(x_253, 1); - x_256 = x_253; -} else { - lean_dec_ref(x_253); - x_256 = lean_box(0); -} -x_257 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_209); -x_258 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__9; -x_259 = l_Lean_Meta_Linear_Nat_reflTrue; -x_260 = l_Lean_mkApp3(x_258, x_254, x_257, x_259); -x_261 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__12; -x_262 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_262, 0, x_261); -lean_ctor_set(x_262, 1, x_260); -if (lean_is_scalar(x_210)) { - x_263 = lean_alloc_ctor(1, 1, 0); +x_250 = lean_ctor_get(x_224, 0); +lean_inc(x_250); +x_251 = lean_ctor_get(x_224, 1); +lean_inc(x_251); +if (lean_is_exclusive(x_224)) { + lean_ctor_release(x_224, 0); + lean_ctor_release(x_224, 1); + x_252 = x_224; } else { - x_263 = x_210; + lean_dec_ref(x_224); + x_252 = lean_box(0); } -lean_ctor_set(x_263, 0, x_262); -if (lean_is_scalar(x_256)) { - x_264 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_252)) { + x_253 = lean_alloc_ctor(1, 2, 0); } else { - x_264 = x_256; -} -lean_ctor_set(x_264, 0, x_263); -lean_ctor_set(x_264, 1, x_255); -return x_264; + x_253 = x_252; } -else -{ -lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; -lean_dec(x_210); -lean_dec(x_209); -x_265 = lean_ctor_get(x_253, 0); -lean_inc(x_265); -x_266 = lean_ctor_get(x_253, 1); -lean_inc(x_266); -if (lean_is_exclusive(x_253)) { - lean_ctor_release(x_253, 0); - lean_ctor_release(x_253, 1); - x_267 = x_253; -} else { - lean_dec_ref(x_253); - x_267 = lean_box(0); +lean_ctor_set(x_253, 0, x_250); +lean_ctor_set(x_253, 1, x_251); +return x_253; } -if (lean_is_scalar(x_267)) { - x_268 = lean_alloc_ctor(1, 2, 0); -} else { - x_268 = x_267; } -lean_ctor_set(x_268, 0, x_265); -lean_ctor_set(x_268, 1, x_266); -return x_268; } } } -else +LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: { -lean_object* x_269; -lean_dec(x_212); -lean_dec(x_1); -x_269 = l_Lean_Meta_Linear_Nat_toContextExpr(x_208, x_2, x_3, x_4, x_5, x_17); -if (lean_obj_tag(x_269) == 0) +lean_object* x_7; lean_object* x_8; +x_7 = lean_alloc_closure((void*)(l_Lean_Meta_Linear_Nat_ToLinear_toLinearCnstr_x3f), 7, 1); +lean_closure_set(x_7, 0, x_1); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +x_8 = l_Lean_Meta_Linear_Nat_ToLinear_run___rarg(x_7, x_2, x_3, x_4, x_5, x_6); +if (lean_obj_tag(x_8) == 0) { -lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; -x_270 = lean_ctor_get(x_269, 0); -lean_inc(x_270); -x_271 = lean_ctor_get(x_269, 1); -lean_inc(x_271); -if (lean_is_exclusive(x_269)) { - lean_ctor_release(x_269, 0); - lean_ctor_release(x_269, 1); - x_272 = x_269; -} else { - lean_dec_ref(x_269); - x_272 = lean_box(0); -} -x_273 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_209); -x_274 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__15; -x_275 = l_Lean_Meta_Linear_Nat_reflTrue; -x_276 = l_Lean_mkApp3(x_274, x_270, x_273, x_275); -x_277 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__18; -x_278 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_278, 0, x_277); -lean_ctor_set(x_278, 1, x_276); -if (lean_is_scalar(x_210)) { - x_279 = lean_alloc_ctor(1, 1, 0); -} else { - x_279 = x_210; -} -lean_ctor_set(x_279, 0, x_278); -if (lean_is_scalar(x_272)) { - x_280 = lean_alloc_ctor(0, 2, 0); -} else { - x_280 = x_272; -} -lean_ctor_set(x_280, 0, x_279); -lean_ctor_set(x_280, 1, x_271); -return x_280; +lean_object* x_9; lean_object* x_10; +x_9 = lean_ctor_get(x_8, 0); +lean_inc(x_9); +x_10 = lean_ctor_get(x_9, 0); +lean_inc(x_10); +if (lean_obj_tag(x_10) == 0) +{ +uint8_t x_11; +lean_dec(x_9); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_11 = !lean_is_exclusive(x_8); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; +x_12 = lean_ctor_get(x_8, 0); +lean_dec(x_12); +x_13 = lean_box(0); +lean_ctor_set(x_8, 0, x_13); +return x_8; } else { -lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; -lean_dec(x_210); -lean_dec(x_209); -x_281 = lean_ctor_get(x_269, 0); -lean_inc(x_281); -x_282 = lean_ctor_get(x_269, 1); -lean_inc(x_282); -if (lean_is_exclusive(x_269)) { - lean_ctor_release(x_269, 0); - lean_ctor_release(x_269, 1); - x_283 = x_269; -} else { - lean_dec_ref(x_269); - x_283 = lean_box(0); -} -if (lean_is_scalar(x_283)) { - x_284 = lean_alloc_ctor(1, 2, 0); -} else { - x_284 = x_283; -} -lean_ctor_set(x_284, 0, x_281); -lean_ctor_set(x_284, 1, x_282); -return x_284; -} +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_8, 1); +lean_inc(x_14); +lean_dec(x_8); +x_15 = lean_box(0); +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_16, 1, x_14); +return x_16; } } +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_17 = lean_ctor_get(x_8, 1); +lean_inc(x_17); +lean_dec(x_8); +x_18 = lean_ctor_get(x_9, 1); +lean_inc(x_18); +lean_dec(x_9); +x_19 = lean_ctor_get(x_10, 0); +lean_inc(x_19); +lean_dec(x_10); +x_20 = lean_alloc_closure((void*)(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1), 7, 1); +lean_closure_set(x_20, 0, x_19); +x_21 = l_Lean_Meta_Linear_Nat_withAbstractAtoms(x_18, x_20, x_2, x_3, x_4, x_5, x_17); +return x_21; } } else { -uint8_t x_285; +uint8_t x_22; lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_285 = !lean_is_exclusive(x_8); -if (x_285 == 0) +x_22 = !lean_is_exclusive(x_8); +if (x_22 == 0) { return x_8; } else { -lean_object* x_286; lean_object* x_287; lean_object* x_288; -x_286 = lean_ctor_get(x_8, 0); -x_287 = lean_ctor_get(x_8, 1); -lean_inc(x_287); -lean_inc(x_286); +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_8, 0); +x_24 = lean_ctor_get(x_8, 1); +lean_inc(x_24); +lean_inc(x_23); lean_dec(x_8); -x_288 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_288, 0, x_286); -lean_ctor_set(x_288, 1, x_287); -return x_288; +x_25 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +return x_25; } } } @@ -2225,7 +3072,7 @@ static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__16() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__1; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__1; x_2 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__15; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; @@ -2243,7 +3090,7 @@ static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__18() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__1; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__1; x_2 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__17; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; @@ -2270,7 +3117,7 @@ static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__21() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__1; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__1; x_2 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__20; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; @@ -2288,7 +3135,7 @@ static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__23() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__1; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__1; x_2 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__22; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; @@ -2719,10 +3566,10 @@ static lean_object* _init_l_Lean_Meta_Linear_Nat_simpExpr_x3f___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__1; -x_2 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__2; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__1; +x_2 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__1; x_3 = l_Lean_Meta_Linear_Nat_simpExpr_x3f___closed__1; -x_4 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__4; +x_4 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__3; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } @@ -3184,42 +4031,54 @@ _G_initialized = true; res = initialize_Lean_Meta_Tactic_LinearArith_Nat_Basic(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__1 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__1(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__1); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__2 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__2(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__2); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__3 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__3(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__3); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__4 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__4(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__4); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__5 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__5(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__5); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__6 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__6(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__6); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__7 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__7(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__7); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__8 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__8(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__8); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__9 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__9(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__9); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__10 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__10(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__10); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__11 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__11(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__11); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__12 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__12(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__12); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__13 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__13(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__13); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__14 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__14(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__14); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__15 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__15(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__15); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__16 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__16(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__16); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__17 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__17(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__17); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__18 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__18(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__18); +l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__1 = _init_l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__1(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__1); +l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__2 = _init_l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__2(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__2); +l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__3 = _init_l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__3(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__3); +l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__1 = _init_l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__1(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__1); +l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__2 = _init_l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__2(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__2); +l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__3 = _init_l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__3(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__3); +l_Lean_Meta_withLocalDecls___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__4___rarg___closed__1 = _init_l_Lean_Meta_withLocalDecls___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__4___rarg___closed__1(); +lean_mark_persistent(l_Lean_Meta_withLocalDecls___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__4___rarg___closed__1); +l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__1 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__1); +l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__2 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__2); +l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__3 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__3); +l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__4 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__4); +l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__5 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__5); +l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__6 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__6); +l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__7 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__7(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__7); +l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__8 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__8(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__8); +l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__9 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__9(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__9); +l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__10 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__10(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__10); +l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__11 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__11(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__11); +l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__12 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__12(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__12); +l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__13 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__13(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__13); +l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__14 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__14(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__14); +l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__15 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__15(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__15); +l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__16 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__16(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__16); +l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__17 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__17(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__17); l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___closed__1 = _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___closed__1(); lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___closed__1); l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___closed__2 = _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___closed__2(); diff --git a/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Solver.c b/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Solver.c index 6e668222227c..20ced03d6778 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Solver.c +++ b/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Solver.c @@ -19,6 +19,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Linear_instDecidableEqCnstrKind___boxed(lea LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprVar____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_166_(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_instReprVar___closed__1; uint8_t l___private_Lean_Data_Rat_0__Lean_beqRat____x40_Lean_Data_Rat___hyg_36_(lean_object*, lean_object*); +lean_object* l_Array_take___rarg(lean_object*, lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_instReprCnstr; static lean_object* l_Lean_Meta_Linear_pickAssignment_x3f___closed__2; @@ -112,6 +113,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Cnstr_getBound___boxed(lean_object*, static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprVar____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_166____closed__10; lean_object* lean_nat_to_int(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_Linear_getBestBound_x3f___spec__1(lean_object*, uint8_t, uint8_t, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Assignment_take(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3803____closed__4; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqPoly____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_420____boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Poly_combine___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -167,6 +169,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean LEAN_EXPORT lean_object* l_Lean_Meta_Linear_instInhabitedAssignment; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Assignment_size(lean_object*); lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Assignment_take___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_decEqAssumptionId____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_2806____boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_beqCnstr____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_4261____boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprVar____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_166____closed__5; @@ -191,7 +194,6 @@ static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta LEAN_EXPORT lean_object* l_Lean_Meta_Linear_State_getNumVars(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_instReprCnstrKind; static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3803____closed__14; -LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Assignment_shrink___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprCnstrKind____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_3803____closed__13; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Poly_combine_go___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_ordVar____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_25_(lean_object*, lean_object*); @@ -208,7 +210,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Poly_getMaxVar(lean_object*); lean_object* lean_int_mul(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Poly_scale___spec__1(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_CnstrKind_toCtorIdx___boxed(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Assignment_shrink(lean_object*, lean_object*); lean_object* lean_string_length(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Solver_0__Lean_Meta_Linear_reprAssumptionId____x40_Lean_Meta_Tactic_LinearArith_Solver___hyg_2896____boxed(lean_object*, lean_object*); lean_object* l_Int_instDecidableEq___boxed(lean_object*, lean_object*); @@ -227,7 +228,6 @@ lean_object* l_instDecidableEqProd___rarg(lean_object*, lean_object*, lean_objec LEAN_EXPORT lean_object* l_Lean_Meta_Linear_instLTVar; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_State_getBestLowerBound_x3f___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Cnstr_isStrict___boxed(lean_object*); -lean_object* l_Array_shrink___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_instReprCnstr___closed__1; uint8_t l_Lean_Rat_lt(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_pickAssignment_x3f___closed__1; @@ -711,19 +711,19 @@ x_3 = lean_array_push(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Assignment_shrink(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Assignment_take(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Array_shrink___rarg(x_1, x_2); +x_3 = l_Array_take___rarg(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Assignment_shrink___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Assignment_take___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Lean_Meta_Linear_Assignment_shrink(x_1, x_2); +x_3 = l_Lean_Meta_Linear_Assignment_take(x_1, x_2); lean_dec(x_2); return x_3; } @@ -5616,7 +5616,7 @@ lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean x_36 = lean_ctor_get(x_1, 0); x_37 = lean_ctor_get(x_1, 1); x_38 = lean_ctor_get(x_1, 3); -x_39 = l_Array_shrink___rarg(x_38, x_34); +x_39 = l_Array_take___rarg(x_38, x_34); x_40 = lean_ctor_get(x_33, 0); lean_inc(x_40); lean_dec(x_33); @@ -5700,7 +5700,7 @@ lean_inc(x_63); lean_inc(x_62); lean_inc(x_61); lean_dec(x_1); -x_65 = l_Array_shrink___rarg(x_64, x_34); +x_65 = l_Array_take___rarg(x_64, x_34); x_66 = lean_ctor_get(x_33, 0); lean_inc(x_66); lean_dec(x_33); diff --git a/stage0/stdlib/Lean/Meta/Tactic/SplitIf.c b/stage0/stdlib/Lean/Meta/Tactic/SplitIf.c index f912d4a7a065..614c73219b72 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/SplitIf.c +++ b/stage0/stdlib/Lean/Meta/Tactic/SplitIf.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Lean.Meta.Tactic.SplitIf -// Imports: Lean.LazyInitExtension Lean.Meta.Tactic.Cases Lean.Meta.Tactic.Simp.Main +// Imports: Lean.Meta.Tactic.Cases Lean.Meta.Tactic.Simp.Main #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -14,18 +14,20 @@ extern "C" { #endif static lean_object* l_Array_findSomeRevM_x3f_find___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___spec__3___closed__5; +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__11; lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -static lean_object* l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__5; -static lean_object* l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__5; +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__9; static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___closed__12; +static lean_object* l_Lean_Meta_SplitIf_getSimpContext___closed__11; static lean_object* l_Lean_Meta_simpIfTarget___closed__9; -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__8; LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_splitIfLocalDecl_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__2; lean_object* lean_mk_empty_array_with_capacity(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_simpIfLocalDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___closed__9; uint8_t l_Lean_Expr_isDIte(lean_object*); +static lean_object* l_Lean_Meta_SplitIf_getSimpContext___closed__8; static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___closed__4; LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_findSomeRevM_x3f_find___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___spec__3___closed__4; @@ -43,85 +45,80 @@ LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at___private_Lean_Meta_ uint8_t l_Lean_Expr_isAppOfArity(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_LocalContext_findDeclRevM_x3f___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_simpIfLocalDecl___closed__1; -static lean_object* l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__2; +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__10; LEAN_EXPORT lean_object* l_Lean_commitWhenSome_x3f___at_Lean_Meta_splitIfLocalDecl_x3f___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_LocalContext_findDeclRevM_x3f___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_SplitIf_splitIfAt_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_SplitIf_mkDischarge_x3f___elambda__1(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__7; +static lean_object* l_Lean_Meta_SplitIf_getSimpContext___closed__10; lean_object* lean_array_fget(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635_(lean_object*); lean_object* l_Lean_MVarId_byCasesDec(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_instantiateMVars___at_Lean_Meta_Simp_synthesizeArgs___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__4; static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___closed__7; static lean_object* l_Lean_Meta_simpIfTarget___closed__11; LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_findIfToSplit_x3f___lambda__1(lean_object*); -lean_object* l_Lean_registerLazyInitExtension___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Meta_SplitIf_splitIfAt_x3f___lambda__2___closed__1; static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___closed__10; lean_object* l_Lean_stringToMessageData(lean_object*); static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___lambda__2___closed__5; static lean_object* l_Array_findSomeRevM_x3f_find___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___spec__3___closed__3; +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__12; static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___closed__8; +static lean_object* l_Lean_Meta_SplitIf_getSimpContext___closed__9; +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__14; static lean_object* l_Lean_Meta_simpIfTarget___closed__6; lean_object* l_Lean_Meta_getSimpCongrTheorems___rarg(lean_object*, lean_object*); lean_object* l_Lean_Expr_appArg_x21(lean_object*); static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___lambda__2___closed__6; -LEAN_EXPORT lean_object* l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4_(lean_object*); static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___lambda__2___closed__1; static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___closed__5; lean_object* l_Lean_LocalDecl_index(lean_object*); static lean_object* l_Array_findSomeRevM_x3f_find___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___spec__3___closed__2; uint8_t l_Lean_Expr_hasMVar(lean_object*); lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_EnvExtension_getState___rarg(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__5; static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___lambda__2___closed__4; -static lean_object* l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__3; +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__1; extern lean_object* l_Lean_PersistentHashMap_empty___at_Lean_Meta_instInhabitedSimpTheorems___spec__1; static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___closed__1; -lean_object* lean_st_ref_take(lean_object*, lean_object*); lean_object* l_Lean_Expr_getRevArg_x21(lean_object*, lean_object*); -static lean_object* l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__7; +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__5; static lean_object* l_Lean_Meta_simpIfTarget___closed__3; static lean_object* l_Lean_Meta_simpIfTarget___closed__8; +static lean_object* l_Lean_Meta_SplitIf_getSimpContext___closed__12; +static uint32_t l_Lean_Meta_SplitIf_getSimpContext___closed__14; static lean_object* l_Lean_Meta_simpIfTarget___closed__5; lean_object* l_Lean_MVarId_getType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_registerTraceClass(lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_findSomeRevM_x3f___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_SplitIf_getSimpContext___closed__3; static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_findIfToSplit_x3f___lambda__1___closed__2; lean_object* l_Lean_Meta_SavedState_restore(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__11; lean_object* l___private_Lean_CoreM_0__Lean_Core_mkFreshNameImp(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_SplitIf_splitIfAt_x3f___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_simpIfTarget___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_findSomeRevM_x3f_find___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___spec__3___closed__1; lean_object* l_Lean_MessageData_ofFormat(lean_object*); -static lean_object* l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__2; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MVarId_withContext___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_synthPendingImp___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_simpTarget(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_DiscrTree_empty(lean_object*); -lean_object* lean_st_ref_get(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_splitIfTarget_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_SplitIf_splitIfAt_x3f___closed__2; LEAN_EXPORT lean_object* l_Lean_PersistentArray_findSomeRevMAux___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_splitIfLocalDecl_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_SplitIf_splitIfAt_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__7; uint8_t l_Lean_Expr_hasLooseBVars(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_SplitIf_ext; LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_SplitIf_getSimpContext(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_isTracingEnabledFor___at_Lean_Meta_Simp_congrArgs___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___lambda__2___closed__2; static lean_object* l_Lean_Meta_simpIfLocalDecl___closed__2; +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__6; LEAN_EXPORT lean_object* l_Lean_Meta_SplitIf_mkDischarge_x3f(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkDecide(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__6; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_findIfToSplit_x3f___boxed(lean_object*); uint8_t lean_name_eq(lean_object*, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); @@ -131,67 +128,56 @@ LEAN_EXPORT lean_object* l_Lean_Meta_SplitIf_mkDischarge_x3f___elambda__1___boxe LEAN_EXPORT lean_object* l_Lean_Meta_simpIfTarget(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isIte(lean_object*); -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__6; lean_object* l_Lean_Meta_saveState___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__4; uint8_t l_Lean_LocalDecl_isAuxDecl(lean_object*); -static lean_object* l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__4; static lean_object* l_Lean_Meta_simpIfTarget___closed__2; static lean_object* l_Lean_Meta_SplitIf_getSimpContext___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_SplitIf_mkDischarge_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofExpr(lean_object*); -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__14; static lean_object* l_Lean_Meta_simpIfTarget___closed__7; -static lean_object* l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__1; -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__10; LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__3; -static lean_object* l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__6; -LEAN_EXPORT lean_object* l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611_(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_findIfToSplit_x3f(lean_object*); static lean_object* l_Lean_Meta_simpIfTarget___closed__10; uint8_t lean_nat_dec_eq(lean_object*, lean_object*); lean_object* l_Lean_mkApp3(lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_EnvExtension_setState___rarg(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_instantiateMVars___at___private_Lean_Meta_Basic_0__Lean_Meta_isClassApp_x3f___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__1; -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__3; lean_object* l_Lean_Meta_mkEqRefl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isConstOf(lean_object*, lean_object*); static lean_object* l_Lean_Meta_simpIfTarget___closed__4; lean_object* l_Lean_LocalDecl_type(lean_object*); -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__9; -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__4; lean_object* l_Lean_addTrace___at_Lean_Meta_Simp_congrArgs___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__2; lean_object* lean_nat_sub(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___lambda__2___closed__3; -static lean_object* l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__3; static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_findIfToSplit_x3f___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_commitWhenSome_x3f___at_Lean_Meta_splitIfTarget_x3f___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); lean_object* l_Lean_Meta_SimpTheorems_addConst(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_SplitIf_getSimpContext___closed__7; lean_object* lean_array_mk(lean_object*); LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_SplitIf_getSimpContext___closed__6; extern lean_object* l_Lean_Meta_Simp_defaultMaxSteps; uint8_t l_Lean_Expr_hasFVar(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___lambda__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_fvar___override(lean_object*); -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__13; +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__13; lean_object* l_Lean_Meta_simpLocalDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addTrace___at_Lean_Meta_processPostponed_loop___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__8; lean_object* lean_local_ctx_num_indices(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_SplitIf_splitIfAt_x3f___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_SplitIf_getSimpContext___closed__5; LEAN_EXPORT lean_object* l_Lean_PersistentArray_findSomeRevMAux___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___closed__3; -static uint32_t l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__8; static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___closed__13; extern lean_object* l_Lean_PersistentHashMap_empty___at_Lean_KeyedDeclsAttribute_instInhabitedExtensionState___spec__1; static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_findIfToSplit_x3f___closed__1; lean_object* l_Lean_isTracingEnabledFor___at_Lean_Meta_processPostponed_loop___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__2; lean_object* lean_array_get_size(lean_object*); lean_object* l_Lean_LocalDecl_toExpr(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_findSomeRevM_x3f___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -199,20 +185,81 @@ lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_obje lean_object* lean_find_expr(lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_findIfToSplit_x3f___lambda__1___boxed(lean_object*); -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__12; -static lean_object* l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__1; static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___lambda__2___closed__7; +static lean_object* l_Lean_Meta_SplitIf_getSimpContext___closed__4; uint8_t l_Lean_Exception_isRuntime(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__15; -static lean_object* l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__3; +static lean_object* l_Lean_Meta_SplitIf_getSimpContext___closed__13; +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__15; LEAN_EXPORT lean_object* l_Lean_Meta_SplitIf_splitIfAt_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_SplitIf_getSimpContext___closed__2; lean_object* l_panic___at_Lean_Meta_subst_substEq___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__4; static lean_object* l_Lean_Meta_simpIfTarget___closed__1; static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___closed__6; static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_findIfToSplit_x3f___closed__3; -static lean_object* _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Meta_SplitIf_getSimpContext___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Meta_DiscrTree_empty(lean_box(0)); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_SplitIf_getSimpContext___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_box(0), lean_box(0)); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_SplitIf_getSimpContext___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Meta_SplitIf_getSimpContext___closed__2; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Meta_SplitIf_getSimpContext___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Meta_SplitIf_getSimpContext___closed__1; +x_2 = l_Lean_PersistentHashMap_empty___at_Lean_Meta_instInhabitedSimpTheorems___spec__1; +x_3 = l_Lean_PersistentHashMap_empty___at_Lean_KeyedDeclsAttribute_instInhabitedExtensionState___spec__1; +x_4 = l_Lean_Meta_SplitIf_getSimpContext___closed__3; +x_5 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_5, 0, x_1); +lean_ctor_set(x_5, 1, x_1); +lean_ctor_set(x_5, 2, x_2); +lean_ctor_set(x_5, 3, x_3); +lean_ctor_set(x_5, 4, x_2); +lean_ctor_set(x_5, 5, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_SplitIf_getSimpContext___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("if_pos", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_SplitIf_getSimpContext___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_SplitIf_getSimpContext___closed__5; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_SplitIf_getSimpContext___closed__7() { _start: { lean_object* x_1; @@ -220,17 +267,17 @@ x_1 = lean_mk_string_unchecked("if_neg", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__2() { +static lean_object* _init_l_Lean_Meta_SplitIf_getSimpContext___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__1; +x_2 = l_Lean_Meta_SplitIf_getSimpContext___closed__7; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__3() { +static lean_object* _init_l_Lean_Meta_SplitIf_getSimpContext___closed__9() { _start: { lean_object* x_1; @@ -238,17 +285,17 @@ x_1 = lean_mk_string_unchecked("dif_pos", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__4() { +static lean_object* _init_l_Lean_Meta_SplitIf_getSimpContext___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__3; +x_2 = l_Lean_Meta_SplitIf_getSimpContext___closed__9; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__5() { +static lean_object* _init_l_Lean_Meta_SplitIf_getSimpContext___closed__11() { _start: { lean_object* x_1; @@ -256,17 +303,17 @@ x_1 = lean_mk_string_unchecked("dif_neg", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__6() { +static lean_object* _init_l_Lean_Meta_SplitIf_getSimpContext___closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__5; +x_2 = l_Lean_Meta_SplitIf_getSimpContext___closed__11; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__7() { +static lean_object* _init_l_Lean_Meta_SplitIf_getSimpContext___closed__13() { _start: { lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; uint8_t x_5; lean_object* x_6; @@ -300,7 +347,7 @@ lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 18, x_4); return x_6; } } -static uint32_t _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__8() { +static uint32_t _init_l_Lean_Meta_SplitIf_getSimpContext___closed__14() { _start: { lean_object* x_1; uint32_t x_2; @@ -309,18 +356,20 @@ x_2 = l_UInt32_ofNatTruncate(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Meta_SplitIf_getSimpContext(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -uint8_t x_8; uint8_t x_9; lean_object* x_10; lean_object* x_11; +lean_object* x_6; lean_object* x_7; uint8_t x_8; uint8_t x_9; lean_object* x_10; lean_object* x_11; +x_6 = l_Lean_Meta_SplitIf_getSimpContext___closed__4; +x_7 = l_Lean_Meta_SplitIf_getSimpContext___closed__6; x_8 = 1; x_9 = 0; x_10 = lean_unsigned_to_nat(1000u); -lean_inc(x_6); -lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -x_11 = l_Lean_Meta_SimpTheorems_addConst(x_1, x_2, x_8, x_9, x_10, x_3, x_4, x_5, x_6, x_7); +lean_inc(x_2); +lean_inc(x_1); +x_11 = l_Lean_Meta_SimpTheorems_addConst(x_6, x_7, x_8, x_9, x_10, x_1, x_2, x_3, x_4, x_5); if (lean_obj_tag(x_11) == 0) { lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; @@ -329,12 +378,12 @@ lean_inc(x_12); x_13 = lean_ctor_get(x_11, 1); lean_inc(x_13); lean_dec(x_11); -x_14 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__2; -lean_inc(x_6); -lean_inc(x_5); +x_14 = l_Lean_Meta_SplitIf_getSimpContext___closed__8; lean_inc(x_4); lean_inc(x_3); -x_15 = l_Lean_Meta_SimpTheorems_addConst(x_12, x_14, x_8, x_9, x_10, x_3, x_4, x_5, x_6, x_13); +lean_inc(x_2); +lean_inc(x_1); +x_15 = l_Lean_Meta_SimpTheorems_addConst(x_12, x_14, x_8, x_9, x_10, x_1, x_2, x_3, x_4, x_13); if (lean_obj_tag(x_15) == 0) { lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; @@ -343,12 +392,12 @@ lean_inc(x_16); x_17 = lean_ctor_get(x_15, 1); lean_inc(x_17); lean_dec(x_15); -x_18 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__4; -lean_inc(x_6); -lean_inc(x_5); +x_18 = l_Lean_Meta_SplitIf_getSimpContext___closed__10; lean_inc(x_4); lean_inc(x_3); -x_19 = l_Lean_Meta_SimpTheorems_addConst(x_16, x_18, x_8, x_9, x_10, x_3, x_4, x_5, x_6, x_17); +lean_inc(x_2); +lean_inc(x_1); +x_19 = l_Lean_Meta_SimpTheorems_addConst(x_16, x_18, x_8, x_9, x_10, x_1, x_2, x_3, x_4, x_17); if (lean_obj_tag(x_19) == 0) { lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; @@ -357,9 +406,9 @@ lean_inc(x_20); x_21 = lean_ctor_get(x_19, 1); lean_inc(x_21); lean_dec(x_19); -x_22 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__6; -lean_inc(x_6); -x_23 = l_Lean_Meta_SimpTheorems_addConst(x_20, x_22, x_8, x_9, x_10, x_3, x_4, x_5, x_6, x_21); +x_22 = l_Lean_Meta_SplitIf_getSimpContext___closed__12; +lean_inc(x_4); +x_23 = l_Lean_Meta_SimpTheorems_addConst(x_20, x_22, x_8, x_9, x_10, x_1, x_2, x_3, x_4, x_21); if (lean_obj_tag(x_23) == 0) { lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; @@ -368,8 +417,8 @@ lean_inc(x_24); x_25 = lean_ctor_get(x_23, 1); lean_inc(x_25); lean_dec(x_23); -x_26 = l_Lean_Meta_getSimpCongrTheorems___rarg(x_6, x_25); -lean_dec(x_6); +x_26 = l_Lean_Meta_getSimpCongrTheorems___rarg(x_4, x_25); +lean_dec(x_4); x_27 = !lean_is_exclusive(x_26); if (x_27 == 0) { @@ -382,8 +431,8 @@ lean_ctor_set(x_30, 1, x_29); x_31 = lean_array_mk(x_30); x_32 = lean_box(0); x_33 = 0; -x_34 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__7; -x_35 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__8; +x_34 = l_Lean_Meta_SplitIf_getSimpContext___closed__13; +x_35 = l_Lean_Meta_SplitIf_getSimpContext___closed__14; x_36 = lean_unsigned_to_nat(0u); x_37 = lean_alloc_ctor(0, 5, 9); lean_ctor_set(x_37, 0, x_34); @@ -412,8 +461,8 @@ lean_ctor_set(x_41, 1, x_40); x_42 = lean_array_mk(x_41); x_43 = lean_box(0); x_44 = 0; -x_45 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__7; -x_46 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__8; +x_45 = l_Lean_Meta_SplitIf_getSimpContext___closed__13; +x_46 = l_Lean_Meta_SplitIf_getSimpContext___closed__14; x_47 = lean_unsigned_to_nat(0u); x_48 = lean_alloc_ctor(0, 5, 9); lean_ctor_set(x_48, 0, x_45); @@ -433,7 +482,7 @@ return x_49; else { uint8_t x_50; -lean_dec(x_6); +lean_dec(x_4); x_50 = !lean_is_exclusive(x_23); if (x_50 == 0) { @@ -457,10 +506,10 @@ return x_53; else { uint8_t x_54; -lean_dec(x_6); -lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); x_54 = !lean_is_exclusive(x_19); if (x_54 == 0) { @@ -484,10 +533,10 @@ return x_57; else { uint8_t x_58; -lean_dec(x_6); -lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); x_58 = !lean_is_exclusive(x_15); if (x_58 == 0) { @@ -509,644 +558,31 @@ return x_61; } } else -{ -uint8_t x_62; -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_62 = !lean_is_exclusive(x_11); -if (x_62 == 0) -{ -return x_11; -} -else -{ -lean_object* x_63; lean_object* x_64; lean_object* x_65; -x_63 = lean_ctor_get(x_11, 0); -x_64 = lean_ctor_get(x_11, 1); -lean_inc(x_64); -lean_inc(x_63); -lean_dec(x_11); -x_65 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_65, 0, x_63); -lean_ctor_set(x_65, 1, x_64); -return x_65; -} -} -} -} -static lean_object* _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__1() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_Meta_DiscrTree_empty(lean_box(0)); -return x_1; -} -} -static lean_object* _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__2() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_box(0), lean_box(0)); -return x_1; -} -} -static lean_object* _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__2; -x_2 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__1; -x_2 = l_Lean_PersistentHashMap_empty___at_Lean_Meta_instInhabitedSimpTheorems___spec__1; -x_3 = l_Lean_PersistentHashMap_empty___at_Lean_KeyedDeclsAttribute_instInhabitedExtensionState___spec__1; -x_4 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__3; -x_5 = lean_alloc_ctor(0, 6, 0); -lean_ctor_set(x_5, 0, x_1); -lean_ctor_set(x_5, 1, x_1); -lean_ctor_set(x_5, 2, x_2); -lean_ctor_set(x_5, 3, x_3); -lean_ctor_set(x_5, 4, x_2); -lean_ctor_set(x_5, 5, x_4); -return x_5; -} -} -static lean_object* _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__5() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("if_pos", 6, 6); -return x_1; -} -} -static lean_object* _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__5; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4_(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_2 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__4; -x_3 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__6; -x_4 = lean_alloc_closure((void*)(l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1), 7, 2); -lean_closure_set(x_4, 0, x_2); -lean_closure_set(x_4, 1, x_3); -x_5 = l_Lean_registerLazyInitExtension___rarg(x_4, x_1); -return x_5; -} -} -static lean_object* _init_l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__3; -x_2 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_2, 0, x_1); -lean_ctor_set(x_2, 1, x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__3; -x_2 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_2, 0, x_1); -lean_ctor_set(x_2, 1, x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__3; -x_2 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_2, 0, x_1); -lean_ctor_set(x_2, 1, x_1); -lean_ctor_set(x_2, 2, x_1); -lean_ctor_set(x_2, 3, x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__2; -x_2 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__3; -x_3 = l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__3; -x_4 = lean_alloc_ctor(0, 7, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_2); -lean_ctor_set(x_4, 3, x_2); -lean_ctor_set(x_4, 4, x_2); -lean_ctor_set(x_4, 5, x_3); -lean_ctor_set(x_4, 6, x_3); -return x_4; -} -} -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -lean_object* x_7; uint8_t x_8; -x_7 = lean_st_ref_get(x_5, x_6); -x_8 = !lean_is_exclusive(x_7); -if (x_8 == 0) -{ -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_9 = lean_ctor_get(x_7, 0); -x_10 = lean_ctor_get(x_7, 1); -x_11 = lean_ctor_get(x_9, 0); -lean_inc(x_11); -lean_dec(x_9); -x_12 = lean_box(0); -x_13 = lean_ctor_get(x_1, 0); -lean_inc(x_13); -x_14 = l_Lean_EnvExtension_getState___rarg(x_12, x_13, x_11); -lean_dec(x_11); -if (lean_obj_tag(x_14) == 0) -{ -lean_object* x_15; lean_object* x_16; -lean_free_object(x_7); -x_15 = lean_ctor_get(x_1, 1); -lean_inc(x_15); -lean_dec(x_1); -lean_inc(x_5); -lean_inc(x_3); -x_16 = lean_apply_5(x_15, x_2, x_3, x_4, x_5, x_10); -if (lean_obj_tag(x_16) == 0) -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_16, 1); -lean_inc(x_18); -lean_dec(x_16); -x_19 = lean_st_ref_take(x_5, x_18); -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_19, 1); -lean_inc(x_21); -lean_dec(x_19); -x_22 = !lean_is_exclusive(x_20); -if (x_22 == 0) -{ -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; -x_23 = lean_ctor_get(x_20, 0); -x_24 = lean_ctor_get(x_20, 4); -lean_dec(x_24); -lean_inc(x_17); -x_25 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_25, 0, x_17); -x_26 = l_Lean_EnvExtension_setState___rarg(x_13, x_23, x_25); -lean_dec(x_13); -x_27 = l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__1; -lean_ctor_set(x_20, 4, x_27); -lean_ctor_set(x_20, 0, x_26); -x_28 = lean_st_ref_set(x_5, x_20, x_21); -lean_dec(x_5); -x_29 = lean_ctor_get(x_28, 1); -lean_inc(x_29); -lean_dec(x_28); -x_30 = lean_st_ref_take(x_3, x_29); -x_31 = lean_ctor_get(x_30, 0); -lean_inc(x_31); -x_32 = lean_ctor_get(x_30, 1); -lean_inc(x_32); -lean_dec(x_30); -x_33 = !lean_is_exclusive(x_31); -if (x_33 == 0) -{ -lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; -x_34 = lean_ctor_get(x_31, 1); -lean_dec(x_34); -x_35 = l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__4; -lean_ctor_set(x_31, 1, x_35); -x_36 = lean_st_ref_set(x_3, x_31, x_32); -lean_dec(x_3); -x_37 = !lean_is_exclusive(x_36); -if (x_37 == 0) -{ -lean_object* x_38; -x_38 = lean_ctor_get(x_36, 0); -lean_dec(x_38); -lean_ctor_set(x_36, 0, x_17); -return x_36; -} -else -{ -lean_object* x_39; lean_object* x_40; -x_39 = lean_ctor_get(x_36, 1); -lean_inc(x_39); -lean_dec(x_36); -x_40 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_40, 0, x_17); -lean_ctor_set(x_40, 1, x_39); -return x_40; -} -} -else -{ -lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_41 = lean_ctor_get(x_31, 0); -x_42 = lean_ctor_get(x_31, 2); -x_43 = lean_ctor_get(x_31, 3); -x_44 = lean_ctor_get(x_31, 4); -lean_inc(x_44); -lean_inc(x_43); -lean_inc(x_42); -lean_inc(x_41); -lean_dec(x_31); -x_45 = l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__4; -x_46 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_46, 0, x_41); -lean_ctor_set(x_46, 1, x_45); -lean_ctor_set(x_46, 2, x_42); -lean_ctor_set(x_46, 3, x_43); -lean_ctor_set(x_46, 4, x_44); -x_47 = lean_st_ref_set(x_3, x_46, x_32); -lean_dec(x_3); -x_48 = lean_ctor_get(x_47, 1); -lean_inc(x_48); -if (lean_is_exclusive(x_47)) { - lean_ctor_release(x_47, 0); - lean_ctor_release(x_47, 1); - x_49 = x_47; -} else { - lean_dec_ref(x_47); - x_49 = lean_box(0); -} -if (lean_is_scalar(x_49)) { - x_50 = lean_alloc_ctor(0, 2, 0); -} else { - x_50 = x_49; -} -lean_ctor_set(x_50, 0, x_17); -lean_ctor_set(x_50, 1, x_48); -return x_50; -} -} -else -{ -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; -x_51 = lean_ctor_get(x_20, 0); -x_52 = lean_ctor_get(x_20, 1); -x_53 = lean_ctor_get(x_20, 2); -x_54 = lean_ctor_get(x_20, 3); -x_55 = lean_ctor_get(x_20, 5); -x_56 = lean_ctor_get(x_20, 6); -lean_inc(x_56); -lean_inc(x_55); -lean_inc(x_54); -lean_inc(x_53); -lean_inc(x_52); -lean_inc(x_51); -lean_dec(x_20); -lean_inc(x_17); -x_57 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_57, 0, x_17); -x_58 = l_Lean_EnvExtension_setState___rarg(x_13, x_51, x_57); -lean_dec(x_13); -x_59 = l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__1; -x_60 = lean_alloc_ctor(0, 7, 0); -lean_ctor_set(x_60, 0, x_58); -lean_ctor_set(x_60, 1, x_52); -lean_ctor_set(x_60, 2, x_53); -lean_ctor_set(x_60, 3, x_54); -lean_ctor_set(x_60, 4, x_59); -lean_ctor_set(x_60, 5, x_55); -lean_ctor_set(x_60, 6, x_56); -x_61 = lean_st_ref_set(x_5, x_60, x_21); -lean_dec(x_5); -x_62 = lean_ctor_get(x_61, 1); -lean_inc(x_62); -lean_dec(x_61); -x_63 = lean_st_ref_take(x_3, x_62); -x_64 = lean_ctor_get(x_63, 0); -lean_inc(x_64); -x_65 = lean_ctor_get(x_63, 1); -lean_inc(x_65); -lean_dec(x_63); -x_66 = lean_ctor_get(x_64, 0); -lean_inc(x_66); -x_67 = lean_ctor_get(x_64, 2); -lean_inc(x_67); -x_68 = lean_ctor_get(x_64, 3); -lean_inc(x_68); -x_69 = lean_ctor_get(x_64, 4); -lean_inc(x_69); -if (lean_is_exclusive(x_64)) { - lean_ctor_release(x_64, 0); - lean_ctor_release(x_64, 1); - lean_ctor_release(x_64, 2); - lean_ctor_release(x_64, 3); - lean_ctor_release(x_64, 4); - x_70 = x_64; -} else { - lean_dec_ref(x_64); - x_70 = lean_box(0); -} -x_71 = l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__4; -if (lean_is_scalar(x_70)) { - x_72 = lean_alloc_ctor(0, 5, 0); -} else { - x_72 = x_70; -} -lean_ctor_set(x_72, 0, x_66); -lean_ctor_set(x_72, 1, x_71); -lean_ctor_set(x_72, 2, x_67); -lean_ctor_set(x_72, 3, x_68); -lean_ctor_set(x_72, 4, x_69); -x_73 = lean_st_ref_set(x_3, x_72, x_65); -lean_dec(x_3); -x_74 = lean_ctor_get(x_73, 1); -lean_inc(x_74); -if (lean_is_exclusive(x_73)) { - lean_ctor_release(x_73, 0); - lean_ctor_release(x_73, 1); - x_75 = x_73; -} else { - lean_dec_ref(x_73); - x_75 = lean_box(0); -} -if (lean_is_scalar(x_75)) { - x_76 = lean_alloc_ctor(0, 2, 0); -} else { - x_76 = x_75; -} -lean_ctor_set(x_76, 0, x_17); -lean_ctor_set(x_76, 1, x_74); -return x_76; -} -} -else -{ -uint8_t x_77; -lean_dec(x_13); -lean_dec(x_5); -lean_dec(x_3); -x_77 = !lean_is_exclusive(x_16); -if (x_77 == 0) -{ -return x_16; -} -else -{ -lean_object* x_78; lean_object* x_79; lean_object* x_80; -x_78 = lean_ctor_get(x_16, 0); -x_79 = lean_ctor_get(x_16, 1); -lean_inc(x_79); -lean_inc(x_78); -lean_dec(x_16); -x_80 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_80, 0, x_78); -lean_ctor_set(x_80, 1, x_79); -return x_80; -} -} -} -else -{ -lean_object* x_81; -lean_dec(x_13); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_81 = lean_ctor_get(x_14, 0); -lean_inc(x_81); -lean_dec(x_14); -lean_ctor_set(x_7, 0, x_81); -return x_7; -} -} -else -{ -lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; -x_82 = lean_ctor_get(x_7, 0); -x_83 = lean_ctor_get(x_7, 1); -lean_inc(x_83); -lean_inc(x_82); -lean_dec(x_7); -x_84 = lean_ctor_get(x_82, 0); -lean_inc(x_84); -lean_dec(x_82); -x_85 = lean_box(0); -x_86 = lean_ctor_get(x_1, 0); -lean_inc(x_86); -x_87 = l_Lean_EnvExtension_getState___rarg(x_85, x_86, x_84); -lean_dec(x_84); -if (lean_obj_tag(x_87) == 0) -{ -lean_object* x_88; lean_object* x_89; -x_88 = lean_ctor_get(x_1, 1); -lean_inc(x_88); -lean_dec(x_1); -lean_inc(x_5); -lean_inc(x_3); -x_89 = lean_apply_5(x_88, x_2, x_3, x_4, x_5, x_83); -if (lean_obj_tag(x_89) == 0) -{ -lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; -x_90 = lean_ctor_get(x_89, 0); -lean_inc(x_90); -x_91 = lean_ctor_get(x_89, 1); -lean_inc(x_91); -lean_dec(x_89); -x_92 = lean_st_ref_take(x_5, x_91); -x_93 = lean_ctor_get(x_92, 0); -lean_inc(x_93); -x_94 = lean_ctor_get(x_92, 1); -lean_inc(x_94); -lean_dec(x_92); -x_95 = lean_ctor_get(x_93, 0); -lean_inc(x_95); -x_96 = lean_ctor_get(x_93, 1); -lean_inc(x_96); -x_97 = lean_ctor_get(x_93, 2); -lean_inc(x_97); -x_98 = lean_ctor_get(x_93, 3); -lean_inc(x_98); -x_99 = lean_ctor_get(x_93, 5); -lean_inc(x_99); -x_100 = lean_ctor_get(x_93, 6); -lean_inc(x_100); -if (lean_is_exclusive(x_93)) { - lean_ctor_release(x_93, 0); - lean_ctor_release(x_93, 1); - lean_ctor_release(x_93, 2); - lean_ctor_release(x_93, 3); - lean_ctor_release(x_93, 4); - lean_ctor_release(x_93, 5); - lean_ctor_release(x_93, 6); - x_101 = x_93; -} else { - lean_dec_ref(x_93); - x_101 = lean_box(0); -} -lean_inc(x_90); -x_102 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_102, 0, x_90); -x_103 = l_Lean_EnvExtension_setState___rarg(x_86, x_95, x_102); -lean_dec(x_86); -x_104 = l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__1; -if (lean_is_scalar(x_101)) { - x_105 = lean_alloc_ctor(0, 7, 0); -} else { - x_105 = x_101; -} -lean_ctor_set(x_105, 0, x_103); -lean_ctor_set(x_105, 1, x_96); -lean_ctor_set(x_105, 2, x_97); -lean_ctor_set(x_105, 3, x_98); -lean_ctor_set(x_105, 4, x_104); -lean_ctor_set(x_105, 5, x_99); -lean_ctor_set(x_105, 6, x_100); -x_106 = lean_st_ref_set(x_5, x_105, x_94); -lean_dec(x_5); -x_107 = lean_ctor_get(x_106, 1); -lean_inc(x_107); -lean_dec(x_106); -x_108 = lean_st_ref_take(x_3, x_107); -x_109 = lean_ctor_get(x_108, 0); -lean_inc(x_109); -x_110 = lean_ctor_get(x_108, 1); -lean_inc(x_110); -lean_dec(x_108); -x_111 = lean_ctor_get(x_109, 0); -lean_inc(x_111); -x_112 = lean_ctor_get(x_109, 2); -lean_inc(x_112); -x_113 = lean_ctor_get(x_109, 3); -lean_inc(x_113); -x_114 = lean_ctor_get(x_109, 4); -lean_inc(x_114); -if (lean_is_exclusive(x_109)) { - lean_ctor_release(x_109, 0); - lean_ctor_release(x_109, 1); - lean_ctor_release(x_109, 2); - lean_ctor_release(x_109, 3); - lean_ctor_release(x_109, 4); - x_115 = x_109; -} else { - lean_dec_ref(x_109); - x_115 = lean_box(0); -} -x_116 = l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__4; -if (lean_is_scalar(x_115)) { - x_117 = lean_alloc_ctor(0, 5, 0); -} else { - x_117 = x_115; -} -lean_ctor_set(x_117, 0, x_111); -lean_ctor_set(x_117, 1, x_116); -lean_ctor_set(x_117, 2, x_112); -lean_ctor_set(x_117, 3, x_113); -lean_ctor_set(x_117, 4, x_114); -x_118 = lean_st_ref_set(x_3, x_117, x_110); -lean_dec(x_3); -x_119 = lean_ctor_get(x_118, 1); -lean_inc(x_119); -if (lean_is_exclusive(x_118)) { - lean_ctor_release(x_118, 0); - lean_ctor_release(x_118, 1); - x_120 = x_118; -} else { - lean_dec_ref(x_118); - x_120 = lean_box(0); -} -if (lean_is_scalar(x_120)) { - x_121 = lean_alloc_ctor(0, 2, 0); -} else { - x_121 = x_120; -} -lean_ctor_set(x_121, 0, x_90); -lean_ctor_set(x_121, 1, x_119); -return x_121; -} -else -{ -lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; -lean_dec(x_86); -lean_dec(x_5); -lean_dec(x_3); -x_122 = lean_ctor_get(x_89, 0); -lean_inc(x_122); -x_123 = lean_ctor_get(x_89, 1); -lean_inc(x_123); -if (lean_is_exclusive(x_89)) { - lean_ctor_release(x_89, 0); - lean_ctor_release(x_89, 1); - x_124 = x_89; -} else { - lean_dec_ref(x_89); - x_124 = lean_box(0); -} -if (lean_is_scalar(x_124)) { - x_125 = lean_alloc_ctor(1, 2, 0); -} else { - x_125 = x_124; -} -lean_ctor_set(x_125, 0, x_122); -lean_ctor_set(x_125, 1, x_123); -return x_125; -} -} -else -{ -lean_object* x_126; lean_object* x_127; -lean_dec(x_86); -lean_dec(x_5); +{ +uint8_t x_62; lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_126 = lean_ctor_get(x_87, 0); -lean_inc(x_126); -lean_dec(x_87); -x_127 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_127, 0, x_126); -lean_ctor_set(x_127, 1, x_83); -return x_127; -} -} -} +x_62 = !lean_is_exclusive(x_11); +if (x_62 == 0) +{ +return x_11; } -static lean_object* _init_l_Lean_Meta_SplitIf_getSimpContext___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = l_Lean_Meta_SplitIf_ext; -return x_1; +lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_63 = lean_ctor_get(x_11, 0); +x_64 = lean_ctor_get(x_11, 1); +lean_inc(x_64); +lean_inc(x_63); +lean_dec(x_11); +x_65 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_65, 0, x_63); +lean_ctor_set(x_65, 1, x_64); +return x_65; } } -LEAN_EXPORT lean_object* l_Lean_Meta_SplitIf_getSimpContext(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; lean_object* x_7; -x_6 = l_Lean_Meta_SplitIf_getSimpContext___closed__1; -x_7 = l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1(x_6, x_1, x_2, x_3, x_4, x_5); -return x_7; } } static lean_object* _init_l_Array_findSomeRevM_x3f_find___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___spec__3___closed__1() { @@ -4131,7 +3567,7 @@ static lean_object* _init_l_Lean_Meta_simpIfTarget___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__3; +x_1 = l_Lean_Meta_SplitIf_getSimpContext___closed__3; x_2 = lean_unsigned_to_nat(0u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -4179,7 +3615,7 @@ static lean_object* _init_l_Lean_Meta_simpIfTarget___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__3; +x_1 = l_Lean_Meta_SplitIf_getSimpContext___closed__3; x_2 = l_Lean_Meta_simpIfTarget___closed__5; x_3 = lean_alloc_ctor(0, 4, 0); lean_ctor_set(x_3, 0, x_1); @@ -4231,7 +3667,7 @@ static lean_object* _init_l_Lean_Meta_simpIfTarget___closed__11() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_simpIfTarget___closed__8; x_2 = l_Lean_Meta_simpIfTarget___closed__9; -x_3 = lean_unsigned_to_nat(101u); +x_3 = lean_unsigned_to_nat(96u); x_4 = lean_unsigned_to_nat(4u); x_5 = l_Lean_Meta_simpIfTarget___closed__10; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -4241,182 +3677,181 @@ return x_6; LEAN_EXPORT lean_object* l_Lean_Meta_simpIfTarget(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { -lean_object* x_8; lean_object* x_9; -x_8 = l_Lean_Meta_SplitIf_getSimpContext___closed__1; +lean_object* x_8; lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -x_9 = l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1(x_8, x_3, x_4, x_5, x_6, x_7); -if (lean_obj_tag(x_9) == 0) +x_8 = l_Lean_Meta_SplitIf_getSimpContext(x_3, x_4, x_5, x_6, x_7); +if (lean_obj_tag(x_8) == 0) { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_10 = lean_ctor_get(x_9, 0); +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_9 = lean_ctor_get(x_8, 0); +lean_inc(x_9); +x_10 = lean_ctor_get(x_8, 1); lean_inc(x_10); -x_11 = lean_ctor_get(x_9, 1); -lean_inc(x_11); -lean_dec(x_9); -x_12 = lean_box(x_2); -x_13 = lean_alloc_closure((void*)(l_Lean_Meta_SplitIf_mkDischarge_x3f___boxed), 6, 1); -lean_closure_set(x_13, 0, x_12); +lean_dec(x_8); +x_11 = lean_box(x_2); +x_12 = lean_alloc_closure((void*)(l_Lean_Meta_SplitIf_mkDischarge_x3f___boxed), 6, 1); +lean_closure_set(x_12, 0, x_11); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_1); -x_14 = l_Lean_MVarId_withContext___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_synthPendingImp___spec__2___rarg(x_1, x_13, x_3, x_4, x_5, x_6, x_11); -if (lean_obj_tag(x_14) == 0) +x_13 = l_Lean_MVarId_withContext___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_synthPendingImp___spec__2___rarg(x_1, x_12, x_3, x_4, x_5, x_6, x_10); +if (lean_obj_tag(x_13) == 0) { -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; -x_15 = lean_ctor_get(x_14, 0); +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; lean_object* x_20; +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_13, 1); lean_inc(x_15); -x_16 = lean_ctor_get(x_14, 1); -lean_inc(x_16); -lean_dec(x_14); -x_17 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_17, 0, x_15); -x_18 = l_Lean_Meta_simpIfTarget___closed__1; -x_19 = 0; -x_20 = l_Lean_Meta_simpIfTarget___closed__7; +lean_dec(x_13); +x_16 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_16, 0, x_14); +x_17 = l_Lean_Meta_simpIfTarget___closed__1; +x_18 = 0; +x_19 = l_Lean_Meta_simpIfTarget___closed__7; lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -x_21 = l_Lean_Meta_simpTarget(x_1, x_10, x_18, x_17, x_19, x_20, x_3, x_4, x_5, x_6, x_16); -if (lean_obj_tag(x_21) == 0) +x_20 = l_Lean_Meta_simpTarget(x_1, x_9, x_17, x_16, x_18, x_19, x_3, x_4, x_5, x_6, x_15); +if (lean_obj_tag(x_20) == 0) { -lean_object* x_22; lean_object* x_23; +lean_object* x_21; lean_object* x_22; +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); x_22 = lean_ctor_get(x_21, 0); lean_inc(x_22); -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -lean_dec(x_22); -if (lean_obj_tag(x_23) == 0) -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_21, 1); -lean_inc(x_24); lean_dec(x_21); -x_25 = l_Lean_Meta_simpIfTarget___closed__11; -x_26 = l_panic___at_Lean_Meta_subst_substEq___spec__1(x_25, x_3, x_4, x_5, x_6, x_24); -return x_26; +if (lean_obj_tag(x_22) == 0) +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_20, 1); +lean_inc(x_23); +lean_dec(x_20); +x_24 = l_Lean_Meta_simpIfTarget___closed__11; +x_25 = l_panic___at_Lean_Meta_subst_substEq___spec__1(x_24, x_3, x_4, x_5, x_6, x_23); +return x_25; } else { -uint8_t x_27; +uint8_t x_26; lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_27 = !lean_is_exclusive(x_21); -if (x_27 == 0) +x_26 = !lean_is_exclusive(x_20); +if (x_26 == 0) { -lean_object* x_28; lean_object* x_29; -x_28 = lean_ctor_get(x_21, 0); -lean_dec(x_28); -x_29 = lean_ctor_get(x_23, 0); -lean_inc(x_29); -lean_dec(x_23); -lean_ctor_set(x_21, 0, x_29); -return x_21; +lean_object* x_27; lean_object* x_28; +x_27 = lean_ctor_get(x_20, 0); +lean_dec(x_27); +x_28 = lean_ctor_get(x_22, 0); +lean_inc(x_28); +lean_dec(x_22); +lean_ctor_set(x_20, 0, x_28); +return x_20; } else { -lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_30 = lean_ctor_get(x_21, 1); +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_20, 1); +lean_inc(x_29); +lean_dec(x_20); +x_30 = lean_ctor_get(x_22, 0); lean_inc(x_30); -lean_dec(x_21); -x_31 = lean_ctor_get(x_23, 0); -lean_inc(x_31); -lean_dec(x_23); -x_32 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_32, 0, x_31); -lean_ctor_set(x_32, 1, x_30); -return x_32; +lean_dec(x_22); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_30); +lean_ctor_set(x_31, 1, x_29); +return x_31; } } } else { -uint8_t x_33; +uint8_t x_32; lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_33 = !lean_is_exclusive(x_21); -if (x_33 == 0) +x_32 = !lean_is_exclusive(x_20); +if (x_32 == 0) { -return x_21; +return x_20; } else { -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_21, 0); -x_35 = lean_ctor_get(x_21, 1); -lean_inc(x_35); +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_20, 0); +x_34 = lean_ctor_get(x_20, 1); lean_inc(x_34); -lean_dec(x_21); -x_36 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_36, 0, x_34); -lean_ctor_set(x_36, 1, x_35); -return x_36; +lean_inc(x_33); +lean_dec(x_20); +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +return x_35; } } } else { -uint8_t x_37; -lean_dec(x_10); +uint8_t x_36; +lean_dec(x_9); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_37 = !lean_is_exclusive(x_14); -if (x_37 == 0) +x_36 = !lean_is_exclusive(x_13); +if (x_36 == 0) { -return x_14; +return x_13; } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_14, 0); -x_39 = lean_ctor_get(x_14, 1); -lean_inc(x_39); +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_13, 0); +x_38 = lean_ctor_get(x_13, 1); lean_inc(x_38); -lean_dec(x_14); -x_40 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_40, 0, x_38); -lean_ctor_set(x_40, 1, x_39); -return x_40; +lean_inc(x_37); +lean_dec(x_13); +x_39 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_39, 0, x_37); +lean_ctor_set(x_39, 1, x_38); +return x_39; } } } else { -uint8_t x_41; +uint8_t x_40; lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_41 = !lean_is_exclusive(x_9); -if (x_41 == 0) +x_40 = !lean_is_exclusive(x_8); +if (x_40 == 0) { -return x_9; +return x_8; } else { -lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_ctor_get(x_9, 0); -x_43 = lean_ctor_get(x_9, 1); -lean_inc(x_43); +lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_41 = lean_ctor_get(x_8, 0); +x_42 = lean_ctor_get(x_8, 1); lean_inc(x_42); -lean_dec(x_9); -x_44 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_44, 0, x_42); -lean_ctor_set(x_44, 1, x_43); -return x_44; +lean_inc(x_41); +lean_dec(x_8); +x_43 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_43, 0, x_41); +lean_ctor_set(x_43, 1, x_42); +return x_43; } } } @@ -4456,7 +3891,7 @@ static lean_object* _init_l_Lean_Meta_simpIfLocalDecl___closed__3() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_simpIfTarget___closed__8; x_2 = l_Lean_Meta_simpIfLocalDecl___closed__2; -x_3 = lean_unsigned_to_nat(108u); +x_3 = lean_unsigned_to_nat(103u); x_4 = lean_unsigned_to_nat(4u); x_5 = l_Lean_Meta_simpIfTarget___closed__10; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -4466,185 +3901,184 @@ return x_6; LEAN_EXPORT lean_object* l_Lean_Meta_simpIfLocalDecl(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { -lean_object* x_8; lean_object* x_9; -x_8 = l_Lean_Meta_SplitIf_getSimpContext___closed__1; +lean_object* x_8; lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -x_9 = l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1(x_8, x_3, x_4, x_5, x_6, x_7); -if (lean_obj_tag(x_9) == 0) +x_8 = l_Lean_Meta_SplitIf_getSimpContext(x_3, x_4, x_5, x_6, x_7); +if (lean_obj_tag(x_8) == 0) { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_10 = lean_ctor_get(x_9, 0); +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_9 = lean_ctor_get(x_8, 0); +lean_inc(x_9); +x_10 = lean_ctor_get(x_8, 1); lean_inc(x_10); -x_11 = lean_ctor_get(x_9, 1); -lean_inc(x_11); -lean_dec(x_9); -x_12 = l_Lean_Meta_simpIfLocalDecl___closed__1; +lean_dec(x_8); +x_11 = l_Lean_Meta_simpIfLocalDecl___closed__1; lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_1); -x_13 = l_Lean_MVarId_withContext___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_synthPendingImp___spec__2___rarg(x_1, x_12, x_3, x_4, x_5, x_6, x_11); -if (lean_obj_tag(x_13) == 0) +x_12 = l_Lean_MVarId_withContext___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_synthPendingImp___spec__2___rarg(x_1, x_11, x_3, x_4, x_5, x_6, x_10); +if (lean_obj_tag(x_12) == 0) { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; lean_object* x_20; -x_14 = lean_ctor_get(x_13, 0); +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; lean_object* x_19; +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_12, 1); lean_inc(x_14); -x_15 = lean_ctor_get(x_13, 1); -lean_inc(x_15); -lean_dec(x_13); -x_16 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_16, 0, x_14); -x_17 = l_Lean_Meta_simpIfTarget___closed__1; -x_18 = 0; -x_19 = l_Lean_Meta_simpIfTarget___closed__7; +lean_dec(x_12); +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_13); +x_16 = l_Lean_Meta_simpIfTarget___closed__1; +x_17 = 0; +x_18 = l_Lean_Meta_simpIfTarget___closed__7; lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -x_20 = l_Lean_Meta_simpLocalDecl(x_1, x_2, x_10, x_17, x_16, x_18, x_19, x_3, x_4, x_5, x_6, x_15); -if (lean_obj_tag(x_20) == 0) +x_19 = l_Lean_Meta_simpLocalDecl(x_1, x_2, x_9, x_16, x_15, x_17, x_18, x_3, x_4, x_5, x_6, x_14); +if (lean_obj_tag(x_19) == 0) { -lean_object* x_21; lean_object* x_22; +lean_object* x_20; lean_object* x_21; +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); x_21 = lean_ctor_get(x_20, 0); lean_inc(x_21); -x_22 = lean_ctor_get(x_21, 0); -lean_inc(x_22); -lean_dec(x_21); -if (lean_obj_tag(x_22) == 0) -{ -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_20, 1); -lean_inc(x_23); lean_dec(x_20); -x_24 = l_Lean_Meta_simpIfLocalDecl___closed__3; -x_25 = l_panic___at_Lean_Meta_subst_substEq___spec__1(x_24, x_3, x_4, x_5, x_6, x_23); -return x_25; +if (lean_obj_tag(x_21) == 0) +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_19, 1); +lean_inc(x_22); +lean_dec(x_19); +x_23 = l_Lean_Meta_simpIfLocalDecl___closed__3; +x_24 = l_panic___at_Lean_Meta_subst_substEq___spec__1(x_23, x_3, x_4, x_5, x_6, x_22); +return x_24; } else { -lean_object* x_26; uint8_t x_27; +lean_object* x_25; uint8_t x_26; lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_26 = lean_ctor_get(x_22, 0); -lean_inc(x_26); -lean_dec(x_22); -x_27 = !lean_is_exclusive(x_20); -if (x_27 == 0) +x_25 = lean_ctor_get(x_21, 0); +lean_inc(x_25); +lean_dec(x_21); +x_26 = !lean_is_exclusive(x_19); +if (x_26 == 0) { -lean_object* x_28; lean_object* x_29; -x_28 = lean_ctor_get(x_20, 0); -lean_dec(x_28); -x_29 = lean_ctor_get(x_26, 1); -lean_inc(x_29); -lean_dec(x_26); -lean_ctor_set(x_20, 0, x_29); -return x_20; +lean_object* x_27; lean_object* x_28; +x_27 = lean_ctor_get(x_19, 0); +lean_dec(x_27); +x_28 = lean_ctor_get(x_25, 1); +lean_inc(x_28); +lean_dec(x_25); +lean_ctor_set(x_19, 0, x_28); +return x_19; } else { -lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_30 = lean_ctor_get(x_20, 1); +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_19, 1); +lean_inc(x_29); +lean_dec(x_19); +x_30 = lean_ctor_get(x_25, 1); lean_inc(x_30); -lean_dec(x_20); -x_31 = lean_ctor_get(x_26, 1); -lean_inc(x_31); -lean_dec(x_26); -x_32 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_32, 0, x_31); -lean_ctor_set(x_32, 1, x_30); -return x_32; +lean_dec(x_25); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_30); +lean_ctor_set(x_31, 1, x_29); +return x_31; } } } else { -uint8_t x_33; +uint8_t x_32; lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_33 = !lean_is_exclusive(x_20); -if (x_33 == 0) +x_32 = !lean_is_exclusive(x_19); +if (x_32 == 0) { -return x_20; +return x_19; } else { -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_20, 0); -x_35 = lean_ctor_get(x_20, 1); -lean_inc(x_35); +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_19, 0); +x_34 = lean_ctor_get(x_19, 1); lean_inc(x_34); -lean_dec(x_20); -x_36 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_36, 0, x_34); -lean_ctor_set(x_36, 1, x_35); -return x_36; +lean_inc(x_33); +lean_dec(x_19); +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +return x_35; } } } else { -uint8_t x_37; -lean_dec(x_10); +uint8_t x_36; +lean_dec(x_9); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_37 = !lean_is_exclusive(x_13); -if (x_37 == 0) +x_36 = !lean_is_exclusive(x_12); +if (x_36 == 0) { -return x_13; +return x_12; } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_13, 0); -x_39 = lean_ctor_get(x_13, 1); -lean_inc(x_39); +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_12, 0); +x_38 = lean_ctor_get(x_12, 1); lean_inc(x_38); -lean_dec(x_13); -x_40 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_40, 0, x_38); -lean_ctor_set(x_40, 1, x_39); -return x_40; +lean_inc(x_37); +lean_dec(x_12); +x_39 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_39, 0, x_37); +lean_ctor_set(x_39, 1, x_38); +return x_39; } } } else { -uint8_t x_41; +uint8_t x_40; lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_41 = !lean_is_exclusive(x_9); -if (x_41 == 0) +x_40 = !lean_is_exclusive(x_8); +if (x_40 == 0) { -return x_9; +return x_8; } else { -lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_ctor_get(x_9, 0); -x_43 = lean_ctor_get(x_9, 1); -lean_inc(x_43); +lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_41 = lean_ctor_get(x_8, 0); +x_42 = lean_ctor_get(x_8, 1); lean_inc(x_42); -lean_dec(x_9); -x_44 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_44, 0, x_42); -lean_ctor_set(x_44, 1, x_43); -return x_44; +lean_inc(x_41); +lean_dec(x_8); +x_43 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_43, 0, x_41); +lean_ctor_set(x_43, 1, x_42); +return x_43; } } } @@ -6912,7 +6346,7 @@ x_12 = l_Lean_commitWhenSome_x3f___at_Lean_Meta_splitIfLocalDecl_x3f___spec__1(x return x_12; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__1() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__1() { _start: { lean_object* x_1; @@ -6920,27 +6354,27 @@ x_1 = lean_mk_string_unchecked("Lean", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__2() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__1; +x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__3() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__2; +x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__2; x_2 = l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__4() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__4() { _start: { lean_object* x_1; @@ -6948,17 +6382,17 @@ x_1 = lean_mk_string_unchecked("initFn", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__5() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__3; -x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__4; +x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__3; +x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__4; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__6() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__6() { _start: { lean_object* x_1; @@ -6966,47 +6400,47 @@ x_1 = lean_mk_string_unchecked("_@", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__7() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__5; -x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__6; +x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__5; +x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__8() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__7; -x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__1; +x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__7; +x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__9() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__8; +x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__8; x_2 = l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__10() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__9; +x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__9; x_2 = l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__11() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__11() { _start: { lean_object* x_1; @@ -7014,17 +6448,17 @@ x_1 = lean_mk_string_unchecked("SplitIf", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__12() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__10; -x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__11; +x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__10; +x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__11; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__13() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__13() { _start: { lean_object* x_1; @@ -7032,38 +6466,37 @@ x_1 = lean_mk_string_unchecked("_hyg", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__14() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__12; -x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__13; +x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__12; +x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__13; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__15() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__14; -x_2 = lean_unsigned_to_nat(1635u); +x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__14; +x_2 = lean_unsigned_to_nat(1611u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611_(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; x_2 = l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___closed__4; x_3 = 0; -x_4 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__15; +x_4 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__15; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); return x_5; } } -lean_object* initialize_Lean_LazyInitExtension(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Meta_Tactic_Cases(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Meta_Tactic_Simp_Main(uint8_t builtin, lean_object*); static bool _G_initialized = false; @@ -7071,57 +6504,39 @@ LEAN_EXPORT lean_object* initialize_Lean_Meta_Tactic_SplitIf(uint8_t builtin, le lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Lean_LazyInitExtension(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Lean_Meta_Tactic_Cases(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); res = initialize_Lean_Meta_Tactic_Simp_Main(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__1 = _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__1); -l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__2 = _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__2); -l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__3 = _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__3); -l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__4 = _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__4); -l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__5 = _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__5(); -lean_mark_persistent(l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__5); -l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__6 = _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__6(); -lean_mark_persistent(l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__6); -l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__7 = _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__7(); -lean_mark_persistent(l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__7); -l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__8 = _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__8(); -l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__1 = _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__1(); -lean_mark_persistent(l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__1); -l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__2 = _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__2(); -lean_mark_persistent(l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__2); -l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__3 = _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__3(); -lean_mark_persistent(l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__3); -l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__4 = _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__4(); -lean_mark_persistent(l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__4); -l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__5 = _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__5(); -lean_mark_persistent(l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__5); -l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__6 = _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__6(); -lean_mark_persistent(l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__6); -if (builtin) {res = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4_(lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -l_Lean_Meta_SplitIf_ext = lean_io_result_get_value(res); -lean_mark_persistent(l_Lean_Meta_SplitIf_ext); -lean_dec_ref(res); -}l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__1 = _init_l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__1(); -lean_mark_persistent(l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__1); -l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__2 = _init_l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__2(); -lean_mark_persistent(l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__2); -l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__3 = _init_l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__3(); -lean_mark_persistent(l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__3); -l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__4 = _init_l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__4(); -lean_mark_persistent(l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__4); l_Lean_Meta_SplitIf_getSimpContext___closed__1 = _init_l_Lean_Meta_SplitIf_getSimpContext___closed__1(); lean_mark_persistent(l_Lean_Meta_SplitIf_getSimpContext___closed__1); +l_Lean_Meta_SplitIf_getSimpContext___closed__2 = _init_l_Lean_Meta_SplitIf_getSimpContext___closed__2(); +lean_mark_persistent(l_Lean_Meta_SplitIf_getSimpContext___closed__2); +l_Lean_Meta_SplitIf_getSimpContext___closed__3 = _init_l_Lean_Meta_SplitIf_getSimpContext___closed__3(); +lean_mark_persistent(l_Lean_Meta_SplitIf_getSimpContext___closed__3); +l_Lean_Meta_SplitIf_getSimpContext___closed__4 = _init_l_Lean_Meta_SplitIf_getSimpContext___closed__4(); +lean_mark_persistent(l_Lean_Meta_SplitIf_getSimpContext___closed__4); +l_Lean_Meta_SplitIf_getSimpContext___closed__5 = _init_l_Lean_Meta_SplitIf_getSimpContext___closed__5(); +lean_mark_persistent(l_Lean_Meta_SplitIf_getSimpContext___closed__5); +l_Lean_Meta_SplitIf_getSimpContext___closed__6 = _init_l_Lean_Meta_SplitIf_getSimpContext___closed__6(); +lean_mark_persistent(l_Lean_Meta_SplitIf_getSimpContext___closed__6); +l_Lean_Meta_SplitIf_getSimpContext___closed__7 = _init_l_Lean_Meta_SplitIf_getSimpContext___closed__7(); +lean_mark_persistent(l_Lean_Meta_SplitIf_getSimpContext___closed__7); +l_Lean_Meta_SplitIf_getSimpContext___closed__8 = _init_l_Lean_Meta_SplitIf_getSimpContext___closed__8(); +lean_mark_persistent(l_Lean_Meta_SplitIf_getSimpContext___closed__8); +l_Lean_Meta_SplitIf_getSimpContext___closed__9 = _init_l_Lean_Meta_SplitIf_getSimpContext___closed__9(); +lean_mark_persistent(l_Lean_Meta_SplitIf_getSimpContext___closed__9); +l_Lean_Meta_SplitIf_getSimpContext___closed__10 = _init_l_Lean_Meta_SplitIf_getSimpContext___closed__10(); +lean_mark_persistent(l_Lean_Meta_SplitIf_getSimpContext___closed__10); +l_Lean_Meta_SplitIf_getSimpContext___closed__11 = _init_l_Lean_Meta_SplitIf_getSimpContext___closed__11(); +lean_mark_persistent(l_Lean_Meta_SplitIf_getSimpContext___closed__11); +l_Lean_Meta_SplitIf_getSimpContext___closed__12 = _init_l_Lean_Meta_SplitIf_getSimpContext___closed__12(); +lean_mark_persistent(l_Lean_Meta_SplitIf_getSimpContext___closed__12); +l_Lean_Meta_SplitIf_getSimpContext___closed__13 = _init_l_Lean_Meta_SplitIf_getSimpContext___closed__13(); +lean_mark_persistent(l_Lean_Meta_SplitIf_getSimpContext___closed__13); +l_Lean_Meta_SplitIf_getSimpContext___closed__14 = _init_l_Lean_Meta_SplitIf_getSimpContext___closed__14(); l_Array_findSomeRevM_x3f_find___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___spec__3___closed__1 = _init_l_Array_findSomeRevM_x3f_find___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___spec__3___closed__1(); lean_mark_persistent(l_Array_findSomeRevM_x3f_find___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___spec__3___closed__1); l_Array_findSomeRevM_x3f_find___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___spec__3___closed__2 = _init_l_Array_findSomeRevM_x3f_find___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___spec__3___closed__2(); @@ -7218,37 +6633,37 @@ l_Lean_Meta_simpIfLocalDecl___closed__2 = _init_l_Lean_Meta_simpIfLocalDecl___cl lean_mark_persistent(l_Lean_Meta_simpIfLocalDecl___closed__2); l_Lean_Meta_simpIfLocalDecl___closed__3 = _init_l_Lean_Meta_simpIfLocalDecl___closed__3(); lean_mark_persistent(l_Lean_Meta_simpIfLocalDecl___closed__3); -l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__1 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__1(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__1); -l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__2 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__2(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__2); -l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__3 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__3(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__3); -l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__4 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__4(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__4); -l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__5 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__5(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__5); -l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__6 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__6(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__6); -l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__7 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__7(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__7); -l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__8 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__8(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__8); -l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__9 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__9(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__9); -l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__10 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__10(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__10); -l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__11 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__11(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__11); -l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__12 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__12(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__12); -l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__13 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__13(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__13); -l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__14 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__14(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__14); -l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__15 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__15(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__15); -if (builtin) {res = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635_(lean_io_mk_world()); +l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__1 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__1(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__1); +l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__2 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__2(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__2); +l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__3 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__3(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__3); +l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__4 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__4(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__4); +l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__5 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__5(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__5); +l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__6 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__6(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__6); +l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__7 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__7(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__7); +l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__8 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__8(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__8); +l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__9 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__9(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__9); +l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__10 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__10(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__10); +l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__11 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__11(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__11); +l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__12 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__12(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__12); +l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__13 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__13(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__13); +l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__14 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__14(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__14); +l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__15 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__15(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__15); +if (builtin) {res = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }return lean_io_result_mk_ok(lean_box(0)); diff --git a/stage0/stdlib/Lean/Meta/WHNF.c b/stage0/stdlib/Lean/Meta/WHNF.c index d86180f5a619..d51d9826fcf9 100644 --- a/stage0/stdlib/Lean/Meta/WHNF.c +++ b/stage0/stdlib/Lean/Meta/WHNF.c @@ -26,6 +26,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_unfoldDefinition_x3f___lambda__2___boxed(le LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Meta_getStuckMVar_x3f___spec__5(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_reduceRecMatcher_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_canUnfoldAtMatcher___closed__1; +lean_object* l_Array_take___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Meta_reducePow___lambda__3___closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_reduceBinNatOp___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkNatLit(lean_object*); @@ -96,6 +97,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_lambdaTelescope___at_Lean_Meta_smartUnfoldi lean_object* l_Lean_MetavarContext_getDelayedMVarAssignmentCore_x3f(lean_object*, lean_object*); static lean_object* l_Lean_getConstInfoCtor___at___private_Lean_Meta_WHNF_0__Lean_Meta_toCtorWhenStructure___spec__1___closed__4; static lean_object* l_Lean_withTraceNode___at_Lean_Meta_whnfImp___spec__1___lambda__2___closed__1; +lean_object* l_Lean_RecursorVal_getMajorInduct(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Meta_WHNF_0__Lean_Meta_toCtorWhenK___spec__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_WHNF_0__Lean_Meta_isQuotRecStuck_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_markSmartUnfoldingMatchAlt___closed__2; @@ -470,7 +472,6 @@ static lean_object* l_Lean_isTracingEnabledFor___at_Lean_Meta_reducePow___spec__ LEAN_EXPORT lean_object* l_Lean_Meta_whnfEasyCases___at_Lean_Meta_whnfImp___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Meta_getStuckMVar_x3f___spec__2(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_reduceBinNatOp___lambda__3___closed__12; -lean_object* l_Lean_RecursorVal_getInduct(lean_object*); lean_object* l_Nat_add___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_reduceBinNatOp___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_reduceBinNatOp___lambda__3___closed__4; @@ -580,7 +581,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_getStuckMVar_x3f___lambda__21___boxed(lean_ LEAN_EXPORT lean_object* l_Lean_Meta_reduceBinNatOp___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_indentExpr(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_whnfEasyCases___at_Lean_Meta_whnfCore_go___spec__2___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Array_shrink___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_reduceBinNatPred___lambda__6(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_WHNF_0__Lean_Meta_toCtorWhenK___spec__1(lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Meta_whnfEasyCases___at_Lean_Meta_whnfCore_go___spec__2___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1567,7 +1567,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_1, x_27, x_29); -x_31 = l_Array_shrink___rarg(x_30, x_2); +x_31 = l_Array_take___rarg(x_30, x_2); x_32 = l_Lean_mkAppN(x_23, x_31); lean_dec(x_31); lean_ctor_set(x_12, 0, x_32); @@ -1589,7 +1589,7 @@ x_39 = lean_unsigned_to_nat(1u); x_40 = lean_nat_sub(x_36, x_39); lean_dec(x_36); x_41 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_1, x_38, x_40); -x_42 = l_Array_shrink___rarg(x_41, x_2); +x_42 = l_Array_take___rarg(x_41, x_2); x_43 = l_Lean_mkAppN(x_34, x_42); lean_dec(x_42); x_44 = lean_alloc_ctor(1, 1, 0); @@ -1623,7 +1623,7 @@ x_53 = lean_unsigned_to_nat(1u); x_54 = lean_nat_sub(x_50, x_53); lean_dec(x_50); x_55 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_1, x_52, x_54); -x_56 = l_Array_shrink___rarg(x_55, x_2); +x_56 = l_Array_take___rarg(x_55, x_2); x_57 = l_Lean_mkAppN(x_48, x_56); lean_dec(x_56); if (lean_is_scalar(x_47)) { @@ -1821,7 +1821,8 @@ lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_180; lea x_16 = lean_ctor_get(x_14, 0); x_17 = lean_ctor_get(x_14, 1); x_180 = l_Lean_Expr_getAppFn(x_16); -x_181 = l_Lean_RecursorVal_getInduct(x_1); +lean_inc(x_1); +x_181 = l_Lean_RecursorVal_getMajorInduct(x_1); x_182 = l_Lean_Expr_isConstOf(x_180, x_181); lean_dec(x_181); lean_dec(x_180); @@ -2791,7 +2792,8 @@ lean_inc(x_213); lean_inc(x_212); lean_dec(x_14); x_293 = l_Lean_Expr_getAppFn(x_212); -x_294 = l_Lean_RecursorVal_getInduct(x_1); +lean_inc(x_1); +x_294 = l_Lean_RecursorVal_getMajorInduct(x_1); x_295 = l_Lean_Expr_isConstOf(x_293, x_294); lean_dec(x_294); lean_dec(x_293); @@ -3908,7 +3910,7 @@ lean_dec(x_33); x_37 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_3, x_34, x_36); x_38 = lean_ctor_get(x_30, 3); lean_inc(x_38); -x_39 = l_Array_shrink___rarg(x_37, x_38); +x_39 = l_Array_take___rarg(x_37, x_38); lean_dec(x_38); lean_inc(x_11); x_40 = l_Lean_Expr_const___override(x_28, x_11); @@ -4097,7 +4099,7 @@ lean_dec(x_71); x_75 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_3, x_72, x_74); x_76 = lean_ctor_get(x_68, 3); lean_inc(x_76); -x_77 = l_Array_shrink___rarg(x_75, x_76); +x_77 = l_Array_take___rarg(x_75, x_76); lean_dec(x_76); lean_inc(x_11); x_78 = l_Lean_Expr_const___override(x_66, x_11); @@ -5161,7 +5163,8 @@ lean_inc(x_17); x_18 = lean_ctor_get(x_16, 1); lean_inc(x_18); lean_dec(x_16); -x_19 = l_Lean_RecursorVal_getInduct(x_1); +lean_inc(x_1); +x_19 = l_Lean_RecursorVal_getMajorInduct(x_1); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); diff --git a/stage0/stdlib/Lean/Parser/Basic.c b/stage0/stdlib/Lean/Parser/Basic.c index 6b7b40b64404..e12a933254e3 100644 --- a/stage0/stdlib/Lean/Parser/Basic.c +++ b/stage0/stdlib/Lean/Parser/Basic.c @@ -377,6 +377,7 @@ LEAN_EXPORT lean_object* l_Lean_RBNode_ins___at_Lean_Parser_TokenMap_insert___sp LEAN_EXPORT lean_object* l_Lean_Parser_optionalNoAntiquot(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_dbgTraceState(lean_object*, lean_object*); static lean_object* l_Lean_Parser_stringGapFn___closed__2; +lean_object* l_Lean_Parser_ParserState_takeStack(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_atomic_docString__1(lean_object*); static lean_object* l___private_Lean_Parser_Basic_0__Lean_Parser_reprLeadingIdentBehavior____x40_Lean_Parser_Basic___hyg_8831____closed__9; LEAN_EXPORT lean_object* l_Lean_Parser_checkLinebreakBefore___elambda__1___boxed(lean_object*, lean_object*, lean_object*); @@ -721,7 +722,6 @@ static lean_object* l___private_Lean_Parser_Basic_0__Lean_Parser_reprLeadingIden LEAN_EXPORT 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_identFnAux_parse___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_TokenMap_instInhabited(lean_object*); -lean_object* l_Lean_Parser_ParserState_shrinkStack(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_chFn___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_scientificLitFn(lean_object*, lean_object*); static lean_object* l_Lean_Parser_categoryParserFn___closed__3; @@ -831,6 +831,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_withPosition_docString__1(le static lean_object* l___private_Lean_Parser_Basic_0__Lean_Parser_reprLeadingIdentBehavior____x40_Lean_Parser_Basic___hyg_8831____closed__8; static lean_object* l_Lean_Parser_orelseFnCore___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_checkColEq___elambda__1(lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Parser_SyntaxStack_take(lean_object*, lean_object*); static lean_object* l_Lean_Parser_chFn___closed__1; uint8_t l_Lean_Parser_SyntaxStack_isEmpty(lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_find___at_Lean_Parser_indexed___spec__2(lean_object*); @@ -936,7 +937,6 @@ LEAN_EXPORT lean_object* l_Lean_Parser_checkLinebreakBefore___elambda__1(lean_ob static lean_object* l___regBuiltin_Lean_Parser_checkColGt_docString__1___closed__3; lean_object* l_Lean_Parser_ParserState_mkUnexpectedTokenError(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_strAux___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Parser_SyntaxStack_shrink(lean_object*, lean_object*); static lean_object* l___private_Lean_Parser_Basic_0__Lean_Parser_reprRecoveryContext____x40_Lean_Parser_Basic___hyg_1469____closed__14; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_checkColEq_docString__1(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Parser_Basic_0__Lean_Parser_withAntiquotSuffixSpliceFn___lambda__1___boxed(lean_object*, lean_object*, lean_object*); @@ -12488,7 +12488,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_ParserState_keepTop(lean_object* x_1, lea { lean_object* x_3; lean_object* x_4; lean_object* x_5; x_3 = l_Lean_Parser_SyntaxStack_back(x_1); -x_4 = l_Lean_Parser_SyntaxStack_shrink(x_1, x_2); +x_4 = l_Lean_Parser_SyntaxStack_take(x_1, x_2); x_5 = l_Lean_Parser_SyntaxStack_push(x_4, x_3); return x_5; } @@ -12567,7 +12567,7 @@ x_9 = lean_ctor_get(x_1, 2); lean_dec(x_9); x_10 = lean_ctor_get(x_1, 1); lean_dec(x_10); -x_11 = l_Lean_Parser_SyntaxStack_shrink(x_7, x_2); +x_11 = l_Lean_Parser_SyntaxStack_take(x_7, x_2); lean_ctor_set(x_1, 4, x_4); lean_ctor_set(x_1, 2, x_3); lean_ctor_set(x_1, 1, x_5); @@ -12584,7 +12584,7 @@ lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_dec(x_1); -x_15 = l_Lean_Parser_SyntaxStack_shrink(x_12, x_2); +x_15 = l_Lean_Parser_SyntaxStack_take(x_12, x_2); x_16 = lean_alloc_ctor(0, 6, 0); lean_ctor_set(x_16, 0, x_15); lean_ctor_set(x_16, 1, x_5); @@ -12634,7 +12634,7 @@ x_9 = lean_ctor_get(x_4, 0); lean_inc(x_9); lean_inc(x_3); x_10 = l___private_Lean_Parser_Types_0__Lean_Parser_beqError____x40_Lean_Parser_Types___hyg_440_(x_3, x_9); -x_11 = l_Lean_Parser_SyntaxStack_shrink(x_6, x_2); +x_11 = l_Lean_Parser_SyntaxStack_take(x_6, x_2); if (x_10 == 0) { lean_object* x_12; @@ -12659,7 +12659,7 @@ lean_dec(x_4); lean_inc(x_13); lean_inc(x_3); x_14 = l___private_Lean_Parser_Types_0__Lean_Parser_beqError____x40_Lean_Parser_Types___hyg_440_(x_3, x_13); -x_15 = l_Lean_Parser_SyntaxStack_shrink(x_6, x_2); +x_15 = l_Lean_Parser_SyntaxStack_take(x_6, x_2); if (x_14 == 0) { lean_object* x_16; lean_object* x_17; @@ -12708,7 +12708,7 @@ if (lean_is_exclusive(x_4)) { lean_inc(x_24); lean_inc(x_3); x_26 = l___private_Lean_Parser_Types_0__Lean_Parser_beqError____x40_Lean_Parser_Types___hyg_440_(x_3, x_24); -x_27 = l_Lean_Parser_SyntaxStack_shrink(x_19, x_2); +x_27 = l_Lean_Parser_SyntaxStack_take(x_19, x_2); if (x_26 == 0) { lean_object* x_28; lean_object* x_29; lean_object* x_30; @@ -12868,7 +12868,7 @@ x_13 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_O if (x_13 == 0) { lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_14 = l_Lean_Parser_ParserState_shrinkStack(x_6, x_3); +x_14 = l_Lean_Parser_ParserState_takeStack(x_6, x_3); x_15 = lean_box(0); x_16 = l_Lean_Parser_ParserState_pushSyntax(x_14, x_15); return x_16; diff --git a/stage0/stdlib/Lean/Parser/Command.c b/stage0/stdlib/Lean/Parser/Command.c index ec0a9399ac07..b9d73a2736da 100644 --- a/stage0/stdlib/Lean/Parser/Command.c +++ b/stage0/stdlib/Lean/Parser/Command.c @@ -26,6 +26,7 @@ static lean_object* l_Lean_Parser_Command_computedFields___closed__13; static lean_object* l_Lean_Parser_Command_derivingClasses___closed__6; static lean_object* l_Lean_Parser_Command_declValSimple___closed__12; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_universe_declRange__1(lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__6; lean_object* l_Lean_Parser_many1_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_register__tactic__tag_formatter___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_initialize_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -40,6 +41,7 @@ static lean_object* l_Lean_Parser_Tactic_open___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_declModifiersT_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_openHiding_formatter___closed__4; static lean_object* l_Lean_Parser_Command_declId_formatter___closed__11; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__53; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_moduleDoc_parenthesizer__1(lean_object*); static lean_object* l_Lean_Parser_Command_nonrec_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_deriving_formatter___closed__8; @@ -58,6 +60,7 @@ static lean_object* l_Lean_Parser_Tactic_open_formatter___closed__5; static lean_object* l_Lean_Parser_Command_structure___closed__11; static lean_object* l_Lean_Parser_Command_optDefDeriving_parenthesizer___closed__5; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_quot_declRange__1(lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__15; LEAN_EXPORT lean_object* l_Lean_Parser_Command_declId_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_initialize_declRange__1___closed__6; static lean_object* l_Lean_Parser_Command_openSimple___closed__6; @@ -79,7 +82,6 @@ lean_object* l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(lean_object*, lean_obj static lean_object* l___regBuiltin_Lean_Parser_Command_attribute_declRange__1___closed__6; static lean_object* l_Lean_Parser_Command_exit_parenthesizer___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_structImplicitBinder; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__49; LEAN_EXPORT lean_object* l_Lean_Parser_Command_include; static lean_object* l_Lean_Parser_Command_printEqns_formatter___closed__1; static lean_object* l_Lean_Parser_Command_end___closed__4; @@ -148,11 +150,11 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_eoi; static lean_object* l_Lean_Parser_Command_declSig_formatter___closed__1; static lean_object* l_Lean_Parser_Command_axiom_formatter___closed__4; static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__5; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__48; static lean_object* l_Lean_Parser_Command_import___closed__1; static lean_object* l_Lean_Parser_Command_ctor_parenthesizer___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Command_open_declRange__1___closed__2; lean_object* l_Lean_Parser_Term_matchAlts_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__23; static lean_object* l_Lean_Parser_Command_instance___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Command_include_formatter__1___closed__2; static lean_object* l_Lean_Parser_Command_variable_formatter___closed__5; @@ -160,7 +162,6 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_whereStructInst_formatter static lean_object* l_Lean_Parser_Command_namedPrio___closed__10; static lean_object* l___regBuiltin_Lean_Parser_Command_end_parenthesizer__1___closed__2; static lean_object* l_Lean_Parser_Command_whereStructInst___closed__4; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__17; LEAN_EXPORT lean_object* l_Lean_Parser_Command_classTk; static lean_object* l___regBuiltin_Lean_Parser_Command_deriving_formatter__1___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_tactic__extension_declRange__1___closed__6; @@ -190,6 +191,7 @@ static lean_object* l_Lean_Parser_Command_extends_parenthesizer___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Command_structureTk_parenthesizer__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_in; static lean_object* l_Lean_Parser_Command_computedField_formatter___closed__5; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__52; static lean_object* l_Lean_Parser_Command_theorem_parenthesizer___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Command_mutual_declRange__1___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Command_universe_formatter__1___closed__2; @@ -209,7 +211,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_import_parenthesizer__1__ lean_object* l_Lean_Parser_Term_attrInstance_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_check__failure_formatter__1___closed__1; lean_object* l_Lean_addBuiltinDocString(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_version_parenthesizer__1___closed__2; static lean_object* l_Lean_Parser_Command_declSig_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Command_computedFields_formatter__1___closed__1; lean_object* l_Lean_Parser_mkAntiquot_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -261,6 +263,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_moduleDoc_formatter_ static lean_object* l_Lean_Parser_Command_namedPrio___closed__6; static lean_object* l_Lean_Parser_Command_printTacTags_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_tactic__extension___closed__7; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__20; static lean_object* l_Lean_Parser_Command_structImplicitBinder___closed__11; static lean_object* l_Lean_Parser_Command_universe_formatter___closed__2; lean_object* l_Lean_PrettyPrinter_Formatter_orelse_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -269,8 +272,10 @@ static lean_object* l_Lean_Parser_Command_openSimple___closed__2; lean_object* l_Lean_Parser_Term_whereDecls_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_section; static lean_object* l___regBuiltin_Lean_Parser_Command_register__tactic__tag_declRange__1___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_version_formatter__1___closed__1; static lean_object* l_Lean_Parser_Command_addDocString___closed__3; static lean_object* l_Lean_Parser_Command_moduleDoc_formatter___closed__8; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__50; static lean_object* l___regBuiltin_Lean_Parser_Command_eval_docString__1___closed__1; static lean_object* l_Lean_Parser_Command_noncomputable_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_tactic__extension_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -279,13 +284,12 @@ static lean_object* l_Lean_Parser_Command_openOnly_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_variable_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Command_structExplicitBinder___closed__18; static lean_object* l___regBuiltin_Lean_Parser_Command_addDocString_declRange__1___closed__2; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__54; static lean_object* l_Lean_Parser_Command_set__option___closed__4; static lean_object* l_Lean_Parser_Command_print___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Command_export_declRange__1___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_version_formatter__1___closed__2; static lean_object* l_Lean_Parser_Command_declValSimple_parenthesizer___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Command_noncomputableSection_declRange__1___closed__5; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__25; static lean_object* l___regBuiltin_Lean_Parser_Command_structure_formatter__1___closed__1; static lean_object* l_Lean_Parser_Command_structExplicitBinder_formatter___closed__13; static lean_object* l___regBuiltin_Lean_Parser_Command_eval_declRange__1___closed__6; @@ -300,7 +304,6 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems LEAN_EXPORT lean_object* l_Lean_Parser_Command_declModifiers_parenthesizer(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_inductive_formatter___closed__14; static lean_object* l_Lean_Parser_Command_structure_parenthesizer___closed__9; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__13; static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__15; static lean_object* l___regBuiltin_Lean_Parser_Command_printAxioms_declRange__1___closed__2; static lean_object* l_Lean_Parser_Command_abbrev___closed__9; @@ -366,6 +369,7 @@ static lean_object* l_Lean_Parser_Command_structImplicitBinder_parenthesizer___c static lean_object* l_Lean_Parser_Command_declSig___closed__9; static lean_object* l_Lean_Parser_Command_optDefDeriving_formatter___closed__6; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_omit_parenthesizer__1(lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__36; static lean_object* l_Lean_Parser_Command_deriving___closed__11; static lean_object* l_Lean_Parser_Command_structFields_formatter___closed__6; static lean_object* l_Lean_Parser_Command_structSimpleBinder_formatter___closed__3; @@ -385,6 +389,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_eraseAttr_formatter(lean_object*, static lean_object* l_Lean_Parser_Command_whereStructInst___closed__20; static lean_object* l___regBuiltin_Lean_Parser_Command_opaque_formatter__1___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_moduleDoc_declRange__1___closed__4; +LEAN_EXPORT lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3092_(lean_object*); static lean_object* l_Lean_Parser_Command_synth_formatter___closed__2; static lean_object* l_Lean_Parser_Command_declaration_formatter___closed__12; static lean_object* l_Lean_Parser_Command_theorem___closed__9; @@ -482,7 +487,6 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_openHiding_parenthesizer_ static lean_object* l___regBuiltin_Lean_Parser_Term_quot__1___closed__1; static lean_object* l_Lean_Parser_Command_initialize_parenthesizer___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_ctor; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__27; static lean_object* l_Lean_Parser_Command_init__quot___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Command_variable_parenthesizer__1___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_export_declRange__1___closed__4; @@ -525,7 +529,6 @@ static lean_object* l_Lean_Parser_Term_quot_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_declModifiers_parenthesizer___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Command_declModifiers_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_attribute_parenthesizer___closed__10; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__40; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_ctor_parenthesizer__1(lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_noncomputable_formatter__1(lean_object*); static lean_object* l_Lean_Parser_Command_instance___closed__8; @@ -583,6 +586,7 @@ static lean_object* l_Lean_Parser_Command_moduleDoc___closed__4; static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__10; static lean_object* l_Lean_Parser_Command_noncomputableSection_formatter___closed__7; static lean_object* l_Lean_Parser_Command_open___closed__2; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__26; lean_object* l_instDecidableEqChar___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_quot_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Command_abbrev_formatter___closed__5; @@ -594,6 +598,7 @@ static lean_object* l_Lean_Parser_Command_structExplicitBinder_formatter___close static lean_object* l_Lean_Parser_Command_structInstBinder___closed__9; static lean_object* l___regBuiltin_Lean_Parser_Term_precheckedQuot_declRange__1___closed__3; static lean_object* l_Lean_Parser_Command_openRenaming___closed__4; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__11; static lean_object* l_Lean_Parser_Command_moduleDoc_formatter___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_docString__1___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_noncomputableSection_declRange__1___closed__2; @@ -611,6 +616,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_printAxioms_declRange__1_ static lean_object* l_Lean_Parser_Command_end___closed__3; static lean_object* l_Lean_Parser_Command_register__tactic__tag_formatter___closed__2; static lean_object* l_Lean_Parser_Command_computedField___closed__1; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__44; static lean_object* l_Lean_Parser_Command_nonrec___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Term_quot_declRange__1___closed__2; static lean_object* l_Lean_Parser_Command_openRenamingItem_parenthesizer___closed__2; @@ -624,7 +630,6 @@ static lean_object* l_Lean_Parser_Command_tactic__extension___closed__3; static lean_object* l_Lean_Parser_Command_whereStructField_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Tactic_open_parenthesizer__1___closed__1; static lean_object* l_Lean_Parser_Command_whereStructInst___closed__11; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__47; LEAN_EXPORT lean_object* l_Lean_Parser_Command_print; static lean_object* l_Lean_Parser_Term_precheckedQuot___closed__4; static lean_object* l_Lean_Parser_Command_abbrev_parenthesizer___closed__7; @@ -652,10 +657,11 @@ static lean_object* l_Lean_Parser_Command_noncomputableSection___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Command_register__tactic__tag_parenthesizer__1___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_variable_parenthesizer__1(lean_object*); static lean_object* l_Lean_Parser_Command_structImplicitBinder_parenthesizer___closed__2; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__38; LEAN_EXPORT lean_object* l_Lean_Parser_Command_structureTk_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structFields_formatter__1(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_ctor_formatter__1___closed__1; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__44; static lean_object* l_Lean_Parser_Command_structImplicitBinder_formatter___closed__8; static lean_object* l_Lean_Parser_Command_derivingClasses___closed__5; static lean_object* l_Lean_Parser_Command_optDefDeriving_parenthesizer___closed__7; @@ -668,6 +674,7 @@ lean_object* l_Lean_Parser_andthenFn(lean_object*, lean_object*, lean_object*, l static lean_object* l_Lean_Parser_Tactic_set__option_formatter___closed__2; static lean_object* l_Lean_Parser_Command_classInductive___closed__11; static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__4; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__45; static lean_object* l_Lean_Parser_Command_genInjectiveTheorems___closed__6; static lean_object* l_Lean_Parser_Command_instance___closed__1; static lean_object* l_Lean_Parser_Command_whereStructInst_formatter___closed__3; @@ -679,6 +686,7 @@ static lean_object* l_Lean_Parser_Command_namedPrio___closed__4; static lean_object* l_Lean_Parser_Command_declModifiers___closed__4; static lean_object* l_Lean_Parser_Command_register__tactic__tag_formatter___closed__7; lean_object* l_Lean_Parser_withOpenFn(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__51; lean_object* l_Lean_Parser_withOpen_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_abbrev___closed__8; static lean_object* l_Lean_Parser_Command_theorem_formatter___closed__2; @@ -779,6 +787,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_namespace_declRange__1___ static lean_object* l_Lean_Parser_Command_declId___closed__14; LEAN_EXPORT lean_object* l_Lean_Parser_Command_optDeriving_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_nonrec_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__5; static lean_object* l_Lean_Parser_Command_optNamedPrio___closed__1; static lean_object* l_Lean_Parser_Command_printAxioms___closed__4; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_import_formatter__1(lean_object*); @@ -791,6 +800,7 @@ static lean_object* l_Lean_Parser_Command_nonrec_formatter___closed__1; static lean_object* l_Lean_Parser_Command_noncomputableSection___closed__4; static lean_object* l_Lean_Parser_Command_optDeriving___closed__9; LEAN_EXPORT lean_object* l_Lean_Parser_Command_mutual_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__22; static lean_object* l_Lean_Parser_Command_optDeriving_formatter___closed__2; static lean_object* l_Lean_Parser_Command_quot_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Command_ctor_formatter___closed__11; @@ -837,6 +847,7 @@ static lean_object* l_Lean_Parser_Tactic_set__option___closed__7; lean_object* l_Lean_Name_mkStr5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_check__failure_parenthesizer___closed__2; lean_object* l_Lean_Parser_setExpected(lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__33; static lean_object* l_Lean_Parser_Command_in_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_optDefDeriving_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_include___closed__8; @@ -849,6 +860,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_set__option_declRange__1_ static lean_object* l_Lean_Parser_Command_declaration_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Command_structFields_formatter__1___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Command_exit_formatter__1___closed__2; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__8; static lean_object* l_Lean_Parser_Command_set__option_formatter___closed__6; static lean_object* l_Lean_Parser_Command_declModifiers_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_eoi_formatter___closed__2; @@ -873,11 +885,11 @@ static lean_object* l_Lean_Parser_Command_inductive_formatter___closed__15; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_private_formatter__1(lean_object*); static lean_object* l_Lean_Parser_Command_structExplicitBinder___closed__8; static lean_object* l_Lean_Parser_Command_optDeriving_formatter___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_version_parenthesizer__1(lean_object*); static lean_object* l_Lean_Parser_Command_initialize_formatter___closed__11; static lean_object* l___regBuiltin_Lean_Parser_Command_import_declRange__1___closed__5; static lean_object* l_Lean_Parser_Command_variable___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Command_register__tactic__tag_declRange__1___closed__7; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__2; static lean_object* l_Lean_Parser_Command_derivingClasses___closed__8; static lean_object* l_Lean_Parser_Command_partial_formatter___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structInstBinder_parenthesizer__1(lean_object*); @@ -903,6 +915,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_initialize_parenthesizer_ LEAN_EXPORT lean_object* l_Lean_Parser_Command_declValSimple_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_open___closed__3; static lean_object* l_Lean_Parser_Command_declVal_formatter___closed__3; +static lean_object* l_Lean_Parser_Command_version___closed__1; static lean_object* l_Lean_Parser_Command_structFields_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_printTacTags_formatter___closed__4; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_initialize_formatter__1(lean_object*); @@ -942,9 +955,7 @@ static lean_object* l_Lean_Parser_Command_open_formatter___closed__5; static lean_object* l_Lean_Parser_Term_precheckedQuot___closed__7; static lean_object* l_Lean_Parser_Command_quot___closed__11; static lean_object* l___regBuiltin_Lean_Parser_Command_init__quot_formatter__1___closed__1; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__24; static lean_object* l___regBuiltin_Lean_Parser_Command_classInductive_parenthesizer__1___closed__1; -LEAN_EXPORT lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097_(lean_object*); static lean_object* l_Lean_Parser_Command_printAxioms_parenthesizer___closed__3; lean_object* l_Lean_Parser_priorityParser_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_deriving___closed__8; @@ -953,14 +964,12 @@ static lean_object* l_Lean_Parser_Command_ctor___closed__13; static lean_object* l_Lean_Parser_Command_computedField_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_declaration___closed__8; static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__17; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__31; static lean_object* l_Lean_Parser_Command_check_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_structFields___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Command_end_formatter__1___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_exit__1(lean_object*); static lean_object* l_Lean_Parser_Command_print___closed__9; static lean_object* l_Lean_Parser_Command_computedField___closed__11; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__22; static lean_object* l_Lean_Parser_Command_mutual_parenthesizer___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Term_precheckedQuot_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_universe_declRange__1___closed__5; @@ -1023,7 +1032,6 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_tactic__extension; static lean_object* l_Lean_Parser_Command_openOnly___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_declId_parenthesizer__1(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_exit_declRange__1___closed__6; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__28; static lean_object* l_Lean_Parser_Command_omit___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Command_printEqns_formatter__1___closed__2; static lean_object* l_Lean_Parser_Command_structure___closed__23; @@ -1073,7 +1081,6 @@ static lean_object* l_Lean_Parser_Command_open_formatter___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_synth_parenthesizer__1___closed__2; static lean_object* l_Lean_Parser_Command_structInstBinder___closed__14; static lean_object* l_Lean_Parser_Command_eval___closed__4; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__37; static lean_object* l_Lean_Parser_Command_printEqns_formatter___closed__3; static lean_object* l_Lean_Parser_Command_attribute_formatter___closed__9; static lean_object* l_Lean_Parser_Command_definition_formatter___closed__9; @@ -1146,7 +1153,6 @@ static lean_object* l_Lean_Parser_Command_declValEqns_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_declModifiers_parenthesizer___closed__23; static lean_object* l___regBuiltin_Lean_Parser_Command_declaration_declRange__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Command_tactic__extension_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__46; static lean_object* l_Lean_Parser_Command_derivingClasses_formatter___closed__7; static lean_object* l_Lean_Parser_Term_quot___closed__17; static lean_object* l_Lean_Parser_Command_printEqns___closed__10; @@ -1236,6 +1242,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_structInstBinder_formatte LEAN_EXPORT lean_object* l_Lean_Parser_Command_structFields; static lean_object* l_Lean_Parser_Command_in_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_openScoped_parenthesizer___closed__1; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__24; static lean_object* l_Lean_Parser_Command_genInjectiveTheorems_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_check__failure___closed__8; static lean_object* l___regBuiltin_Lean_Parser_Tactic_set__option_declRange__1___closed__4; @@ -1244,14 +1251,15 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_import_declRange__1___clo static lean_object* l_Lean_Parser_Command_classInductive_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Term_set__option___closed__8; static lean_object* l_Lean_Parser_Command_ctor_parenthesizer___closed__1; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__17; static lean_object* l_Lean_Parser_Command_structure___closed__15; static lean_object* l_Lean_Parser_Command_computedField___closed__7; static lean_object* l_Lean_Parser_Command_optDeriving___closed__2; static lean_object* l_Lean_Parser_Command_optDefDeriving_formatter___closed__4; static lean_object* l_Lean_Parser_Command_attribute___closed__12; static lean_object* l_Lean_Parser_Command_set__option_parenthesizer___closed__8; +static lean_object* l_Lean_Parser_Command_version_parenthesizer___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_whereStructInst_formatter__1(lean_object*); -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__11; static lean_object* l_Lean_Parser_Command_check___closed__8; static lean_object* l_Lean_Parser_Command_extends___closed__1; static lean_object* l_Lean_Parser_Command_declId___closed__19; @@ -1275,6 +1283,7 @@ static lean_object* l_Lean_Parser_Command_optDeriving___closed__7; static lean_object* l_Lean_Parser_Command_declModifiers_parenthesizer___closed__15; static lean_object* l___regBuiltin_Lean_Parser_Command_print_declRange__1___closed__2; static lean_object* l_Lean_Parser_Command_structExplicitBinder___closed__6; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__7; static lean_object* l_Lean_Parser_Command_import_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_structSimpleBinder_formatter___closed__5; static lean_object* l_Lean_Parser_Term_open___closed__1; @@ -1313,7 +1322,6 @@ lean_object* l_Lean_Parser_commandParser_parenthesizer(lean_object*, lean_object static lean_object* l_Lean_Parser_Command_structInstBinder___closed__6; static lean_object* l_Lean_Parser_Command_optDeclSig_formatter___closed__10; static lean_object* l_Lean_Parser_Command_eoi___closed__1; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__30; static lean_object* l_Lean_Parser_Term_set__option___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Command_declModifiers_docString__1___closed__2; static lean_object* l_Lean_Parser_Command_nonrec___closed__4; @@ -1353,7 +1361,6 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_addDocString_declRange__1 static lean_object* l_Lean_Parser_Command_optDefDeriving_parenthesizer___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Command_unsafe_parenthesizer__1___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_end_declRange__1___closed__7; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__51; static lean_object* l_Lean_Parser_Command_optDefDeriving___closed__5; static lean_object* l_Lean_Parser_Command_quot___closed__14; static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__18; @@ -1414,6 +1421,7 @@ static lean_object* l_Lean_Parser_Term_quot___closed__2; static lean_object* l_Lean_Parser_Command_end_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_declSig___closed__6; static lean_object* l_Lean_Parser_Command_moduleDoc_formatter___closed__5; +LEAN_EXPORT lean_object* l_Lean_Parser_Command_version; static lean_object* l_Lean_Parser_Command_whereStructInst___closed__13; static lean_object* l___regBuiltin_Lean_Parser_Command_variable_formatter__1___closed__2; lean_object* l_Lean_Parser_withOpen_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1423,6 +1431,7 @@ static lean_object* l_Lean_Parser_Command_moduleDoc_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_init__quot___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_optDeriving_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_computedFields; +static lean_object* l_Lean_Parser_Command_version_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_mutual_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_classInductive___closed__13; static lean_object* l_Lean_Parser_Command_axiom___closed__4; @@ -1434,6 +1443,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_noncomputableSection static lean_object* l_Lean_Parser_Command_export___closed__3; static lean_object* l_Lean_Parser_Command_opaque___closed__6; static lean_object* l_Lean_Parser_Command_open_parenthesizer___closed__2; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__40; static lean_object* l___regBuiltin_Lean_Parser_Command_whereStructField_formatter__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_derivingClasses; static lean_object* l___regBuiltin_Lean_Parser_Command_deriving_declRange__1___closed__1; @@ -1454,6 +1464,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Tactic_open_declRange__1___closed LEAN_EXPORT lean_object* l_Lean_Parser_Term_precheckedQuot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_partial_parenthesizer__1___closed__2; static lean_object* l_Lean_Parser_Command_universe_formatter___closed__4; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__21; static lean_object* l_Lean_Parser_Command_register__tactic__tag_parenthesizer___closed__4; lean_object* l_Lean_Parser_Term_binderIdent_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_declVal_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1490,6 +1501,7 @@ static lean_object* l_Lean_Parser_Tactic_set__option___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Command_printTacTags_formatter__1___closed__2; static lean_object* l_Lean_Parser_Command_openOnly_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Command_unsafe_formatter__1___closed__2; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__41; static lean_object* l_Lean_Parser_Command_openRenamingItem_formatter___closed__1; static lean_object* l_Lean_Parser_Command_quot___closed__7; static lean_object* l_Lean_Parser_Command_whereStructField___closed__1; @@ -1528,7 +1540,6 @@ static lean_object* l_Lean_Parser_Command_printTacTags___closed__7; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_declaration_declRange__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_check_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_in_parenthesizer__1___closed__2; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__19; static lean_object* l_Lean_Parser_Command_mutual___closed__13; static lean_object* l___regBuiltin_Lean_Parser_Command_open_declRange__1___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Tactic_open_formatter__1___closed__2; @@ -1621,6 +1632,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_deriving__1(lean_obj LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_tactic__extension_declRange__1(lean_object*); static lean_object* l_Lean_Parser_Command_register__tactic__tag_formatter___closed__5; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_whereStructInst_parenthesizer__1(lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__47; static lean_object* l_Lean_Parser_Command_structureTk_formatter___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_openOnly_parenthesizer__1(lean_object*); static lean_object* l_Lean_Parser_Command_structSimpleBinder_formatter___closed__4; @@ -1652,7 +1664,6 @@ static lean_object* l_Lean_Parser_Command_structExplicitBinder_parenthesizer___c static lean_object* l_Lean_Parser_Tactic_open_parenthesizer___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Command_set__option_formatter__1___closed__1; static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__24; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__45; static lean_object* l_Lean_Parser_Command_section_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_protected_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_manyIndent_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1663,11 +1674,10 @@ extern lean_object* l_Lean_Parser_Term_attrKind; static lean_object* l_Lean_Parser_Command_structInstBinder_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_whereStructInst___closed__24; LEAN_EXPORT lean_object* l_Lean_Parser_Command_import_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__42; lean_object* l_Lean_ppLine_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_inductive_formatter__1___closed__1; static lean_object* l_Lean_Parser_Command_structInstBinder___closed__13; -LEAN_EXPORT lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3073_(lean_object*); -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__21; static lean_object* l___regBuiltin_Lean_Parser_Command_unsafe_parenthesizer__1___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_openDecl_docString__1(lean_object*); static lean_object* l_Lean_Parser_Command_register__tactic__tag___closed__7; @@ -1697,6 +1707,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_export_declRange__1___clo static lean_object* l_Lean_Parser_Command_ctor_parenthesizer___closed__5; LEAN_EXPORT uint8_t l_Lean_Parser_Command_declId___lambda__1(uint32_t); static lean_object* l_Lean_Parser_Command_printAxioms___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Command_version_docString__1___closed__1; static lean_object* l_Lean_Parser_Command_register__tactic__tag___closed__3; static lean_object* l_Lean_Parser_Command_addDocString___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Command_set__option_parenthesizer__1___closed__2; @@ -1714,6 +1725,7 @@ LEAN_EXPORT uint8_t l___private_Lean_Parser_Command_0__Lean_Parser_Command_skipU static lean_object* l___regBuiltin_Lean_Parser_Command_structSimpleBinder_formatter__1___closed__1; lean_object* l_Lean_Parser_notFollowedBy(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_structCtor_formatter___closed__2; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__37; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_deriving_declRange__1(lean_object*); static lean_object* l_Lean_Parser_Command_set__option_parenthesizer___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_theorem_formatter__1(lean_object*); @@ -1721,7 +1733,6 @@ static lean_object* l_Lean_Parser_Command_omit_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Command_structureTk_formatter___closed__3; static lean_object* l_Lean_Parser_Command_declBody___closed__5; static lean_object* l_Lean_Parser_Command_abbrev___closed__6; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__34; static lean_object* l_Lean_Parser_Command_noncomputable___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Tactic_open_formatter__1___closed__1; static lean_object* l_Lean_Parser_Command_attribute___closed__7; @@ -1743,7 +1754,6 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_set__option_formatter__1___c static lean_object* l_Lean_Parser_Command_axiom_formatter___closed__5; lean_object* l_Lean_Parser_symbol(lean_object*); static lean_object* l_Lean_Parser_Command_printAxioms_parenthesizer___closed__5; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__9; static lean_object* l_Lean_Parser_Command_namedPrio___closed__11; static lean_object* l___regBuiltin_Lean_Parser_Command_theorem_parenthesizer__1___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_opaque_formatter__1___closed__2; @@ -1751,10 +1761,11 @@ static lean_object* l_Lean_Parser_Command_export_parenthesizer___closed__4; lean_object* l_Lean_Parser_Term_typeSpec_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_precheckedQuot_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_initializeKeyword_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_version___closed__5; static lean_object* l_Lean_Parser_Command_definition_formatter___closed__4; static lean_object* l_Lean_Parser_Command_structFields___closed__13; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__12; static lean_object* l_Lean_Parser_Command_declVal___closed__4; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__32; LEAN_EXPORT lean_object* l_Lean_Parser_Command_addDocString; static lean_object* l_Lean_Parser_Command_structExplicitBinder_formatter___closed__7; static lean_object* l_Lean_Parser_Command_set__option_formatter___closed__1; @@ -1781,7 +1792,6 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_noncomputable_formatter__ extern lean_object* l_Lean_Parser_Tactic_tacticSeq; static lean_object* l_Lean_Parser_Term_quot___closed__3; static lean_object* l_Lean_Parser_Command_declaration_formatter___closed__4; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__15; static lean_object* l___regBuiltin_Lean_Parser_Command_printAxioms_parenthesizer__1___closed__1; static lean_object* l_Lean_Parser_Command_check_formatter___closed__4; static lean_object* l_Lean_Parser_Command_printAxioms___closed__1; @@ -1826,6 +1836,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_quot_parenthesizer__1(l static lean_object* l___regBuiltin_Lean_Parser_Command_inductive_parenthesizer__1___closed__2; static lean_object* l_Lean_Parser_Command_structExplicitBinder___closed__1; static lean_object* l_Lean_Parser_Command_structImplicitBinder_formatter___closed__3; +static lean_object* l_Lean_Parser_Command_version_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_set__option_parenthesizer___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Command_export_parenthesizer__1___closed__1; static lean_object* l_Lean_Parser_Command_universe_parenthesizer___closed__2; @@ -1841,6 +1852,7 @@ static lean_object* l_Lean_Parser_Tactic_open___closed__5; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structExplicitBinder_formatter__1(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_precheckedQuot_parenthesizer__1___closed__2; static lean_object* l_Lean_Parser_Command_derivingClasses_parenthesizer___closed__6; +static lean_object* l_Lean_Parser_Command_version___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Command_register__tactic__tag_declRange__1___closed__2; static lean_object* l_Lean_Parser_Command_partial___closed__3; static lean_object* l_Lean_Parser_Command_moduleDoc___closed__2; @@ -1849,6 +1861,7 @@ static lean_object* l_Lean_Parser_Command_attribute_formatter___closed__4; static lean_object* l_Lean_Parser_Command_structure_parenthesizer___closed__14; static lean_object* l___regBuiltin_Lean_Parser_Command_declaration_declRange__1___closed__2; static lean_object* l_Lean_Parser_Command_noncomputableSection_formatter___closed__1; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__49; static lean_object* l_Lean_Parser_Command_inductive___closed__10; static lean_object* l___regBuiltin_Lean_Parser_Tactic_open__1___closed__2; static lean_object* l_Lean_Parser_Command_printAxioms_parenthesizer___closed__2; @@ -1864,6 +1877,7 @@ static lean_object* l_Lean_Parser_Command_instance_parenthesizer___closed__11; static lean_object* l_Lean_Parser_Command_openRenamingItem_formatter___closed__2; static lean_object* l_Lean_Parser_Command_mutual_parenthesizer___closed__9; static lean_object* l_Lean_Parser_Command_include___closed__3; +static lean_object* l_Lean_Parser_Command_version___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_variable_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_export_formatter___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Command_printAxioms_declRange__1___closed__4; @@ -1882,13 +1896,14 @@ static lean_object* l_Lean_Parser_Command_evalBang___closed__5; static lean_object* l_Lean_Parser_Command_quot_formatter___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Command_noncomputableSection_formatter__1___closed__1; static lean_object* l_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__11; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__12; static lean_object* l_Lean_Parser_Command_openRenaming___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_structCtor; static lean_object* l___regBuiltin_Lean_Parser_Command_abbrev_parenthesizer__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_openDecl_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__29; extern lean_object* l_Lean_Parser_Command_docComment; static lean_object* l_Lean_Parser_Command_openRenaming___closed__12; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__50; static lean_object* l_Lean_Parser_Command_deriving_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_variable_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_tactic__extension_parenthesizer___closed__4; @@ -1920,6 +1935,7 @@ static lean_object* l_Lean_Parser_Command_eoi_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_set__option_declRange__1___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Command_openDecl_docString__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_declBody; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__25; static lean_object* l_Lean_Parser_Command_unsafe_parenthesizer___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_noncomputableSection_parenthesizer__1(lean_object*); static lean_object* l_Lean_Parser_Term_quot_formatter___closed__4; @@ -1965,6 +1981,7 @@ static lean_object* l_Lean_Parser_Command_structFields___closed__11; static lean_object* l_Lean_Parser_Command_ctor_parenthesizer___closed__11; LEAN_EXPORT lean_object* l_Lean_Parser_Command_declModifiersF; static lean_object* l_Lean_Parser_Command_deriving___closed__15; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__9; static lean_object* l_Lean_Parser_Tactic_set__option_formatter___closed__3; static lean_object* l_Lean_Parser_Command_structExplicitBinder___closed__2; static lean_object* l_Lean_Parser_Command_tactic__extension___closed__4; @@ -1981,6 +1998,7 @@ static lean_object* l_Lean_Parser_Command_structure_parenthesizer___closed__15; static lean_object* l_Lean_Parser_Command_attribute___closed__4; static lean_object* l_Lean_Parser_Command_set__option_formatter___closed__3; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_section_parenthesizer__1(lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__54; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_export_formatter__1(lean_object*); static lean_object* l_Lean_Parser_Command_moduleDoc_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_classInductive___closed__15; @@ -2017,7 +2035,6 @@ static lean_object* l_Lean_Parser_Command_initialize___closed__5; static lean_object* l_Lean_Parser_Tactic_open_parenthesizer___closed__3; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_set__option__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_openRenamingItem_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__10; static lean_object* l___regBuiltin_Lean_Parser_Command_deriving_parenthesizer__1___closed__1; lean_object* l_Lean_Parser_Term_attrKind_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_partial___closed__4; @@ -2033,10 +2050,12 @@ static lean_object* l_Lean_Parser_Command_print_parenthesizer___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_declValEqns_formatter__1(lean_object*); static lean_object* l_Lean_Parser_Command_initialize___closed__11; static lean_object* l___regBuiltin_Lean_Parser_Command_initializeKeyword_parenthesizer__1___closed__2; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__46; static lean_object* l___regBuiltin_Lean_Parser_Tactic_set__option_formatter__1___closed__1; static lean_object* l_Lean_Parser_Command_noncomputable_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_genInjectiveTheorems_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_optDeriving___closed__4; +static lean_object* l_Lean_Parser_Command_version___closed__6; static lean_object* l_Lean_Parser_Command_namespace_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_namedPrio_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_declaration_formatter__1___closed__1; @@ -2052,6 +2071,7 @@ static lean_object* l_Lean_Parser_Command_declModifiers_parenthesizer___closed__ lean_object* l_Lean_Parser_many_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_noncomputableSection_parenthesizer___closed__7; lean_object* l_Lean_Parser_Term_attributes_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__10; LEAN_EXPORT lean_object* l_Lean_Parser_Command_structExplicitBinder; static lean_object* l_Lean_Parser_Command_initialize_formatter___closed__5; static lean_object* l_Lean_Parser_Command_optDeclSig_formatter___closed__5; @@ -2073,6 +2093,7 @@ static lean_object* l_Lean_Parser_Command_structureTk___closed__7; static lean_object* l_Lean_Parser_Command_definition_parenthesizer___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Command_deriving_declRange__1___closed__7; static lean_object* l_Lean_Parser_Command_ctor___closed__5; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__13; static lean_object* l___regBuiltin_Lean_Parser_Command_noncomputableSection_formatter__1___closed__2; static lean_object* l_Lean_Parser_Command_axiom___closed__9; static lean_object* l_Lean_Parser_Command_initialize_formatter___closed__1; @@ -2117,7 +2138,6 @@ static lean_object* l_Lean_Parser_Command_openSimple_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_quot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_printTacTags___closed__1; static lean_object* l_Lean_Parser_Command_declValSimple_formatter___closed__10; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__35; static lean_object* l_Lean_Parser_Command_declSig___closed__3; static lean_object* l_Lean_Parser_Command_structure_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_computedFields___closed__12; @@ -2133,6 +2153,7 @@ static lean_object* l_Lean_Parser_Command_instance_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_quot___closed__4; static lean_object* l_Lean_Parser_Command_printTacTags_formatter___closed__5; static lean_object* l_Lean_Parser_Command_optDeclSig_formatter___closed__8; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__28; static lean_object* l_Lean_Parser_Command_structSimpleBinder___closed__1; static lean_object* l_Lean_Parser_Command_opaque___closed__8; static lean_object* l_Lean_Parser_Command_inductive___closed__12; @@ -2313,7 +2334,6 @@ static lean_object* l_Lean_Parser_Command_abbrev___closed__5; static lean_object* l_Lean_Parser_Command_namespace___closed__1; static lean_object* l_Lean_Parser_Command_whereStructInst_formatter___closed__5; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_register__tactic__tag_declRange__1(lean_object*); -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__52; static lean_object* l_Lean_Parser_Command_printTacTags___closed__9; static lean_object* l_Lean_Parser_Command_openRenaming_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_openSimple_formatter__1___closed__2; @@ -2371,6 +2391,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_universe_formatter__ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_declId_formatter__1(lean_object*); static lean_object* l_Lean_Parser_Command_moduleDoc_formatter___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_omit_formatter__1(lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__3; static lean_object* l___regBuiltin_Lean_Parser_Command_declVal_docString__1___closed__3; static lean_object* l_Lean_Parser_Command_opaque_formatter___closed__4; static lean_object* l_Lean_Parser_Command_declaration_parenthesizer___closed__1; @@ -2397,13 +2418,11 @@ static lean_object* l_Lean_Parser_Command_whereStructInst___closed__6; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_declVal_docString__1(lean_object*); static lean_object* l_Lean_Parser_Command_eraseAttr_formatter___closed__3; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_classTk_formatter__1(lean_object*); -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__6; static lean_object* l_Lean_Parser_Command_openHiding_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Command_check__failure_formatter___closed__3; lean_object* l_Lean_Parser_many(lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_openRenamingItem_formatter__1(lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_register__tactic__tag_docString__1(lean_object*); -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__8; static lean_object* l___regBuiltin_Lean_Parser_Command_eoi_parenthesizer__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_synth_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_moduleDoc___closed__3; @@ -2479,6 +2498,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_openSimple_parenthesizer_ static lean_object* l_Lean_Parser_Command_exit_formatter___closed__3; static lean_object* l_Lean_Parser_Command_moduleDoc_parenthesizer___closed__7; lean_object* l_Lean_ppSpace_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__31; LEAN_EXPORT lean_object* l_Lean_Parser_Command_initialize; static lean_object* l_Lean_Parser_Command_openDecl___closed__4; static lean_object* l_Lean_Parser_Command_declValSimple_formatter___closed__4; @@ -2490,6 +2510,7 @@ static lean_object* l_Lean_Parser_Command_extends___closed__9; static lean_object* l___regBuiltin_Lean_Parser_Command_classTk_formatter__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_theorem_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_structImplicitBinder_parenthesizer___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_version_docString__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_import; static lean_object* l_Lean_Parser_Command_noncomputableSection_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_quot_parenthesizer___closed__2; @@ -2536,6 +2557,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_universe_parenthesizer(lean_objec LEAN_EXPORT lean_object* l_Lean_Parser_Command_printTacTags_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_initialize_declRange__1___closed__5; static lean_object* l_Lean_Parser_Tactic_open_parenthesizer___closed__8; +static lean_object* l_Lean_Parser_Command_version___closed__4; static lean_object* l_Lean_Parser_Command_openScoped_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_inductive___closed__4; static lean_object* l_Lean_Parser_Command_attribute___closed__5; @@ -2563,20 +2585,18 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_structInstBinder_formatter(lean_o static lean_object* l___regBuiltin_Lean_Parser_Command_printTacTags_declRange__1___closed__4; static lean_object* l_Lean_Parser_Command_declId_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_classInductive___closed__12; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__20; LEAN_EXPORT lean_object* l_Lean_Parser_Command_namespace_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_namedPrio_parenthesizer___closed__9; static lean_object* l_Lean_Parser_Command_structImplicitBinder_parenthesizer___closed__3; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__53; static lean_object* l___regBuiltin_Lean_Parser_Command_quot_docString__1___closed__1; static lean_object* l_Lean_Parser_Command_declId_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_classTk___closed__5; static lean_object* l_Lean_Parser_Command_tactic__extension_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_nonrec_formatter__1___closed__2; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_set__option_declRange__1___closed__5; static lean_object* l_Lean_Parser_Command_printTacTags___closed__12; lean_object* l_Lean_Parser_sepBy1_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__27; static lean_object* l_Lean_Parser_Command_theorem_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_section_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_optDeriving___closed__6; @@ -2640,11 +2660,12 @@ static lean_object* l_Lean_Parser_Command_eoi_formatter___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_printEqns; static lean_object* l___regBuiltin_Lean_Parser_Command_mutual_parenthesizer__1___closed__1; static lean_object* l_Lean_Parser_Command_tactic__extension___closed__5; +static lean_object* l_Lean_Parser_Command_version___closed__2; static lean_object* l_Lean_Parser_Command_structImplicitBinder___closed__5; static lean_object* l_Lean_Parser_Command_mutual___closed__14; static lean_object* l_Lean_Parser_Command_ctor_parenthesizer___closed__2; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__32; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_theorem_parenthesizer__1(lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_open_declRange__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_eval; static lean_object* l_Lean_Parser_Command_whereStructField___closed__5; @@ -2673,6 +2694,7 @@ static lean_object* l_Lean_Parser_Command_openDecl___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Command_example_parenthesizer__1___closed__2; static lean_object* l_Lean_Parser_Command_definition___closed__12; static lean_object* l_Lean_Parser_Command_definition___closed__5; +LEAN_EXPORT lean_object* l_Lean_Parser_Command_version_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_mutual_parenthesizer___closed__8; LEAN_EXPORT lean_object* l_Lean_Parser_Command_optionValue_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_check__failure_formatter___closed__4; @@ -2745,6 +2767,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Parser_Command_0__Lean_Parser_Command_ extern lean_object* l_Lean_PrettyPrinter_Parenthesizer_parenthesizerAliasesRef; static lean_object* l_Lean_Parser_Command_declValSimple_parenthesizer___closed__7; lean_object* l_Lean_Parser_withAntiquotSpliceAndSuffix(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__35; static lean_object* l_Lean_Parser_Command_evalBang_formatter___closed__4; static lean_object* l_Lean_Parser_Command_set__option_formatter___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Command_quot_formatter__1___closed__2; @@ -2777,7 +2800,6 @@ lean_object* l_Lean_Parser_Term_instBinder_parenthesizer(lean_object*, lean_obje lean_object* l_Lean_Parser_withoutPosition_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_addDocString_formatter___closed__5; static lean_object* l_Lean_Parser_Term_precheckedQuot___closed__2; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__48; static lean_object* l_Lean_Parser_Command_variable___closed__6; static lean_object* l_Lean_Parser_Command_initialize___closed__13; static lean_object* l_Lean_Parser_Command_structExplicitBinder_formatter___closed__12; @@ -2873,6 +2895,7 @@ static lean_object* l_Lean_Parser_Command_export_formatter___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Command_private_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_register__tactic__tag__1(lean_object*); static lean_object* l_Lean_Parser_Command_structFields___closed__16; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__16; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structCtor_parenthesizer__1(lean_object*); static lean_object* l_Lean_Parser_Command_in_formatter___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Command_tactic__extension_declRange__1___closed__7; @@ -2882,6 +2905,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_openRenaming; static lean_object* l___regBuiltin_Lean_Parser_Command_optDeriving_formatter__1___closed__2; static lean_object* l_Lean_Parser_Command_structInstBinder_formatter___closed__6; static lean_object* l_Lean_Parser_Command_openScoped___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_version_formatter__1(lean_object*); static lean_object* l_Lean_Parser_Command_initialize_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Tactic_set__option_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_quot_parenthesizer___closed__3; @@ -2915,12 +2939,10 @@ static lean_object* l_Lean_Parser_Command_open_formatter___closed__2; static lean_object* l_Lean_Parser_Command_axiom___closed__10; static lean_object* l_Lean_Parser_Command_computedField___closed__5; static lean_object* l_Lean_Parser_Command_namedPrio_formatter___closed__6; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__16; LEAN_EXPORT lean_object* l_Lean_Parser_Command_eraseAttr; static lean_object* l_Lean_Parser_Command_declId_formatter___closed__4; static lean_object* l_Lean_Parser_Command_synth___closed__2; static lean_object* l_Lean_Parser_Command_structImplicitBinder___closed__7; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__5; static lean_object* l___regBuiltin_Lean_Parser_Command_init__quot_formatter__1___closed__2; static lean_object* l_Lean_Parser_Command_structure___closed__8; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_end_parenthesizer__1(lean_object*); @@ -2928,13 +2950,11 @@ static lean_object* l_Lean_Parser_Command_eoi_formatter___closed__6; static lean_object* l_Lean_Parser_Command_namedPrio_formatter___closed__2; static lean_object* l_Lean_Parser_Command_openSimple___closed__5; static lean_object* l_Lean_Parser_Command_initialize_formatter___closed__6; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__26; LEAN_EXPORT lean_object* l_Lean_Parser_Command_register__tactic__tag_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_computedField_parenthesizer___closed__8; LEAN_EXPORT lean_object* l_Lean_Parser_Command_namespace_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_structExplicitBinder___closed__16; static lean_object* l_Lean_Parser_Command_namedPrio_formatter___closed__12; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__41; static lean_object* l_Lean_Parser_Command_printAxioms_parenthesizer___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_open_formatter__1(lean_object*); static lean_object* l_Lean_Parser_Command_exit___closed__1; @@ -2993,6 +3013,7 @@ static lean_object* l_Lean_Parser_Command_quot___closed__5; static lean_object* l_Lean_Parser_Command_check___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_protected; static lean_object* l_Lean_Parser_Command_structInstBinder_parenthesizer___closed__2; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__39; static lean_object* l_Lean_Parser_Command_derivingClasses_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_mutual_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_print_formatter___closed__1; @@ -3018,6 +3039,7 @@ static lean_object* l_Lean_Parser_Command_declaration_parenthesizer___closed__3; lean_object* l_Lean_Parser_Tactic_tacticSeq_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_structure_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Term_quot_formatter___closed__6; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__14; static lean_object* l_Lean_Parser_Command_print___closed__10; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_computedFields_parenthesizer__1(lean_object*); static lean_object* l_Lean_Parser_Term_precheckedQuot___closed__8; @@ -3075,12 +3097,11 @@ static lean_object* l_Lean_Parser_Command_derivingClasses_formatter___closed__5; static lean_object* l_Lean_Parser_Command_genInjectiveTheorems___closed__8; static lean_object* l_Lean_Parser_Command_moduleDoc_formatter___closed__3; static lean_object* l_Lean_Parser_Command_import___closed__5; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__42; static lean_object* l_Lean_Parser_Command_namedPrio_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_classTk___closed__1; static lean_object* l_Lean_Parser_Command_set__option___closed__7; static lean_object* l_Lean_Parser_Command_protected_parenthesizer___closed__3; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__4; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__30; LEAN_EXPORT lean_object* l_Lean_Parser_Command_quot; static lean_object* l_Lean_Parser_Command_partial___closed__8; static lean_object* l_Lean_Parser_Command_declId___closed__9; @@ -3095,7 +3116,6 @@ static lean_object* l_Lean_Parser_Command_optDeclSig_formatter___closed__4; static lean_object* l_Lean_Parser_Command_computedFields_formatter___closed__1; lean_object* l_Lean_Parser_Term_bracketedBinder_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_partial; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__33; static lean_object* l_Lean_Parser_Command_abbrev___closed__11; static lean_object* l_Lean_Parser_Command_printEqns_formatter___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Command_printAxioms_formatter__1___closed__1; @@ -3111,6 +3131,7 @@ static lean_object* l_Lean_Parser_Command_structCtor_formatter___closed__6; static lean_object* l_Lean_Parser_Command_optDeclSig___closed__1; static lean_object* l_Lean_Parser_Command_structCtor___closed__5; static lean_object* l_Lean_Parser_Command_mutual_formatter___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_version__1(lean_object*); static lean_object* l_Lean_Parser_Term_quot___closed__18; static lean_object* l___regBuiltin_Lean_Parser_Command_structImplicitBinder_formatter__1___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_namespace_docString__1(lean_object*); @@ -3144,6 +3165,7 @@ static lean_object* l_Lean_Parser_Command_extends_formatter___closed__4; static lean_object* l_Lean_Parser_Command_printEqns___closed__6; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_eval_docString__2(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_openOnly_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__43; static lean_object* l___regBuiltin_Lean_Parser_Term_set__option_parenthesizer__1___closed__1; static lean_object* l_Lean_Parser_Command_omit_formatter___closed__5; static lean_object* l_Lean_Parser_Command_check__failure___closed__3; @@ -3151,6 +3173,7 @@ static lean_object* l_Lean_Parser_Command_classTk___closed__4; static lean_object* l_Lean_Parser_Command_axiom___closed__5; static lean_object* l_Lean_Parser_Term_open_formatter___closed__5; static lean_object* l_Lean_Parser_Command_declModifiers___closed__1; +LEAN_EXPORT lean_object* l_Lean_Parser_Command_version_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_check_formatter__1(lean_object*); static lean_object* l_Lean_Parser_Command_printTacTags_formatter___closed__6; static lean_object* l_Lean_Parser_Command_openRenamingItem___closed__3; @@ -3287,9 +3310,9 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_init__quot_declRange__1__ static lean_object* l_Lean_Parser_Command_import___closed__6; static lean_object* l_Lean_Parser_Command_abbrev_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Command_noncomputable___closed__8; +static lean_object* l_Lean_Parser_Command_version_formatter___closed__2; static lean_object* l_Lean_Parser_Command_opaque_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_inductive_formatter___closed__3; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__29; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_declaration_parenthesizer__1(lean_object*); static lean_object* l_Lean_Parser_Term_open_parenthesizer___closed__4; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_end_docString__1(lean_object*); @@ -3300,6 +3323,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_open_docString__1(lea LEAN_EXPORT lean_object* l_Lean_Parser_Command_universe_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_incQuotDepth_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structImplicitBinder_formatter__1(lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__34; static lean_object* l_Lean_Parser_Command_definition_parenthesizer___closed__9; static lean_object* l___regBuiltin_Lean_Parser_Term_quot_formatter__1___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Command_omit_formatter__1___closed__1; @@ -3324,6 +3348,7 @@ static lean_object* l_Lean_Parser_Command_printEqns_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_declBody___closed__7; static lean_object* l_Lean_Parser_Command_structureTk_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_derivingClasses___closed__1; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__19; LEAN_EXPORT lean_object* l_Lean_Parser_Command_check__failure_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_example_formatter___closed__3; static lean_object* l_Lean_Parser_Command_optionValue_parenthesizer___closed__2; @@ -3351,6 +3376,7 @@ static lean_object* l_Lean_Parser_Command_mutual_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_inductive_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Command_declModifiers_docString__1___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Command_deriving_declRange__1___closed__5; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__23; static lean_object* l_Lean_Parser_Command_ctor___closed__1; static lean_object* l_Lean_Parser_Command_declModifiers___closed__6; static lean_object* l_Lean_Parser_Command_eraseAttr___closed__8; @@ -3361,12 +3387,12 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_declModifiers_formatter(uint8_t, static lean_object* l___regBuiltin_Lean_Parser_Command_export_parenthesizer__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_optionValue; LEAN_EXPORT lean_object* l_Lean_Parser_Command_check; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__36; static lean_object* l_Lean_Parser_Command_structCtor___closed__8; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_mutual_declRange__1(lean_object*); static lean_object* l_Lean_Parser_Command_inductive_formatter___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Command_example_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structureTk_formatter__1(lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__18; static lean_object* l_Lean_Parser_Command_addDocString___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Command_quot_parenthesizer__1___closed__1; static lean_object* l_Lean_Parser_Tactic_set__option___closed__3; @@ -3438,6 +3464,7 @@ static lean_object* l_Lean_Parser_Command_declaration_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Command_import___closed__7; static lean_object* l_Lean_Parser_Command_structExplicitBinder_formatter___closed__6; static lean_object* l_Lean_Parser_Command_declValEqns___closed__3; +static lean_object* l_Lean_Parser_Command_version_formatter___closed__1; static lean_object* l_Lean_Parser_Command_optDefDeriving___closed__11; static lean_object* l_Lean_Parser_Command_classInductive___closed__4; static lean_object* l_Lean_Parser_Command_noncomputable___closed__2; @@ -3518,14 +3545,12 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_unsafe_parenthesizer(lean_object* static lean_object* l_Lean_Parser_Command_tactic__extension___closed__6; static lean_object* l_Lean_Parser_Command_openSimple___closed__3; static lean_object* l_Lean_Parser_Command_eraseAttr_parenthesizer___closed__3; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__38; lean_object* l_Lean_Parser_sepBy1_parenthesizer(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_extends___closed__6; static lean_object* l_Lean_Parser_Command_structExplicitBinder_formatter___closed__11; static lean_object* l_Lean_Parser_Command_noncomputable___closed__1; static lean_object* l_Lean_Parser_Term_open_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_optDeriving_parenthesizer___closed__4; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__7; static lean_object* l_Lean_Parser_Command_register__tactic__tag_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_attribute_formatter___closed__12; static lean_object* l___regBuiltin_Lean_Parser_Term_precheckedQuot_formatter__1___closed__1; @@ -3545,7 +3570,6 @@ static lean_object* l_Lean_Parser_Command_whereStructInst___closed__29; static lean_object* l_Lean_Parser_Command_quot___closed__6; static lean_object* l_Lean_Parser_Command_classInductive___closed__16; static lean_object* l_Lean_Parser_Command_computedFields_parenthesizer___closed__4; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__18; static lean_object* l___regBuiltin_Lean_Parser_Term_set__option_docString__1___closed__1; static lean_object* l_Lean_Parser_Command_inductive_formatter___closed__2; static lean_object* l_Lean_Parser_Command_declSig___closed__2; @@ -3597,10 +3621,10 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structImplicitBinder lean_object* l_Lean_Parser_Term_bracketedBinder(uint8_t); LEAN_EXPORT lean_object* l_Lean_Parser_Command_optDeriving; static lean_object* l_Lean_Parser_Command_declId_parenthesizer___closed__4; +static lean_object* l_Lean_Parser_Command_version_formatter___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_precheckedQuot_declRange__1___closed__1; static lean_object* l_Lean_Parser_Command_openOnly_formatter___closed__5; static lean_object* l_Lean_Parser_Tactic_open_formatter___closed__7; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__14; static lean_object* l_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_attribute___closed__11; static lean_object* l_Lean_Parser_Command_section_parenthesizer___closed__1; @@ -3660,6 +3684,7 @@ static lean_object* l_Lean_Parser_Command_mutual_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_definition_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_computedField_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Command_structSimpleBinder___closed__9; +LEAN_EXPORT lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_print_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_attribute_declRange__1___closed__5; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_partial_parenthesizer__1(lean_object*); @@ -3744,6 +3769,7 @@ static lean_object* l_Lean_Parser_Command_printTacTags___closed__11; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_initializeKeyword_parenthesizer__1(lean_object*); static lean_object* l_Lean_Parser_Command_optDeclSig_formatter___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Command_declValSimple_formatter__1___closed__1; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__4; static lean_object* l___regBuiltin_Lean_Parser_Command_mutual_declRange__1___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Tactic_open_declRange__1___closed__2; static lean_object* l_Lean_Parser_Command_in___closed__1; @@ -3770,13 +3796,12 @@ static lean_object* l_Lean_Parser_Command_evalBang_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_include___closed__1; static lean_object* l_Lean_Parser_Command_variable___closed__10; lean_object* l_Lean_Parser_ppGroup_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_version___closed__8; static lean_object* l_Lean_Parser_Command_attribute___closed__10; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__43; static lean_object* l_Lean_Parser_Command_inductive___closed__15; static lean_object* l_Lean_Parser_Command_set__option_formatter___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Command_include_formatter__1___closed__1; static lean_object* l_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__13; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__39; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_initialize__1(lean_object*); static lean_object* l_Lean_Parser_Command_optDeclSig_formatter___closed__6; static lean_object* l_Lean_Parser_Command_whereStructInst_formatter___closed__10; @@ -3804,6 +3829,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_in__1(lean_object*); static lean_object* l_Lean_Parser_Command_noncomputableSection_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_initialize_formatter__1___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_version_parenthesizer__1___closed__1; static lean_object* l_Lean_Parser_Command_private___closed__6; static lean_object* l_Lean_Parser_Command_definition_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_exit___closed__2; @@ -31185,6 +31211,295 @@ x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); return x_6; } } +static lean_object* _init_l_Lean_Parser_Command_version___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("version", 7, 7); +return x_1; +} +} +static lean_object* _init_l_Lean_Parser_Command_version___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Parser_Term_quot___closed__1; +x_2 = l_Lean_Parser_Term_quot___closed__2; +x_3 = l_Lean_Parser_Command_quot___closed__1; +x_4 = l_Lean_Parser_Command_version___closed__1; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Parser_Command_version___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; +x_1 = l_Lean_Parser_Command_version___closed__1; +x_2 = l_Lean_Parser_Command_version___closed__2; +x_3 = 1; +x_4 = 0; +x_5 = l_Lean_Parser_mkAntiquot(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Parser_Command_version___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("#version", 8, 8); +return x_1; +} +} +static lean_object* _init_l_Lean_Parser_Command_version___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Parser_Command_version___closed__4; +x_2 = l_Lean_Parser_symbol(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Parser_Command_version___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Parser_Command_version___closed__2; +x_2 = lean_unsigned_to_nat(1024u); +x_3 = l_Lean_Parser_Command_version___closed__5; +x_4 = l_Lean_Parser_leadingNode(x_1, x_2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_Parser_Command_version___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_version___closed__3; +x_2 = l_Lean_Parser_Command_version___closed__6; +x_3 = l_Lean_Parser_withAntiquot(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Parser_Command_version___closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_version___closed__2; +x_2 = l_Lean_Parser_Command_version___closed__7; +x_3 = l_Lean_Parser_withCache(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Parser_Command_version() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Parser_Command_version___closed__8; +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_version__1(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_2 = l_Lean_Parser_Command_quot___closed__5; +x_3 = l_Lean_Parser_Command_version___closed__2; +x_4 = 1; +x_5 = l_Lean_Parser_Command_version; +x_6 = lean_unsigned_to_nat(1000u); +x_7 = l_Lean_Parser_addBuiltinParser(x_2, x_3, x_4, x_5, x_6, x_1); +return x_7; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_version_docString__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Shows the current Lean version. Prints `Lean.versionString`. ", 61, 61); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_version_docString__1(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_2 = l_Lean_Parser_Command_version___closed__2; +x_3 = l___regBuiltin_Lean_Parser_Command_version_docString__1___closed__1; +x_4 = l_Lean_addBuiltinDocString(x_2, x_3, x_1); +return x_4; +} +} +static lean_object* _init_l_Lean_Parser_Command_version_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_1 = l_Lean_Parser_Command_version___closed__1; +x_2 = l_Lean_Parser_Command_version___closed__2; +x_3 = 1; +x_4 = 0; +x_5 = lean_box(x_3); +x_6 = lean_box(x_4); +x_7 = lean_alloc_closure((void*)(l_Lean_Parser_mkAntiquot_formatter___boxed), 9, 4); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +lean_closure_set(x_7, 2, x_5); +lean_closure_set(x_7, 3, x_6); +return x_7; +} +} +static lean_object* _init_l_Lean_Parser_Command_version_formatter___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Parser_Command_version___closed__4; +x_2 = lean_alloc_closure((void*)(l_Lean_Parser_symbol_formatter), 6, 1); +lean_closure_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Parser_Command_version_formatter___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Parser_Command_version___closed__2; +x_2 = lean_unsigned_to_nat(1024u); +x_3 = l_Lean_Parser_Command_version_formatter___closed__2; +x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); +lean_closure_set(x_4, 0, x_1); +lean_closure_set(x_4, 1, x_2); +lean_closure_set(x_4, 2, x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Lean_Parser_Command_version_formatter(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_6 = l_Lean_Parser_Command_version_formatter___closed__1; +x_7 = l_Lean_Parser_Command_version_formatter___closed__3; +x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); +return x_8; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_version_formatter__1___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l_Lean_Parser_Term_quot___closed__1; +x_2 = l_Lean_Parser_Term_quot___closed__2; +x_3 = l_Lean_Parser_Command_quot___closed__1; +x_4 = l_Lean_Parser_Command_version___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_quot_formatter__1___closed__1; +x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_version_formatter__1___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_version_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_version_formatter__1(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter__1___closed__3; +x_3 = l_Lean_Parser_Command_version___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_version_formatter__1___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_version_formatter__1___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +static lean_object* _init_l_Lean_Parser_Command_version_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_1 = l_Lean_Parser_Command_version___closed__1; +x_2 = l_Lean_Parser_Command_version___closed__2; +x_3 = 1; +x_4 = 0; +x_5 = lean_box(x_3); +x_6 = lean_box(x_4); +x_7 = lean_alloc_closure((void*)(l_Lean_Parser_mkAntiquot_parenthesizer___boxed), 9, 4); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +lean_closure_set(x_7, 2, x_5); +lean_closure_set(x_7, 3, x_6); +return x_7; +} +} +static lean_object* _init_l_Lean_Parser_Command_version_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Parser_Command_version___closed__4; +x_2 = lean_alloc_closure((void*)(l_Lean_Parser_symbol_parenthesizer), 6, 1); +lean_closure_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Parser_Command_version_parenthesizer___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Parser_Command_version___closed__2; +x_2 = lean_unsigned_to_nat(1024u); +x_3 = l_Lean_Parser_Command_version_parenthesizer___closed__2; +x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer), 8, 3); +lean_closure_set(x_4, 0, x_1); +lean_closure_set(x_4, 1, x_2); +lean_closure_set(x_4, 2, x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Lean_Parser_Command_version_parenthesizer(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_6 = l_Lean_Parser_Command_version_parenthesizer___closed__1; +x_7 = l_Lean_Parser_Command_version_parenthesizer___closed__3; +x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); +return x_8; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_version_parenthesizer__1___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l_Lean_Parser_Term_quot___closed__1; +x_2 = l_Lean_Parser_Term_quot___closed__2; +x_3 = l_Lean_Parser_Command_quot___closed__1; +x_4 = l_Lean_Parser_Command_version___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer__1___closed__1; +x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_version_parenthesizer__1___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_version_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_version_parenthesizer__1(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer__1___closed__3; +x_3 = l_Lean_Parser_Command_version___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_version_parenthesizer__1___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_version_parenthesizer__1___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_init__quot___closed__1() { _start: { @@ -41753,7 +42068,7 @@ x_1 = l_Lean_Parser_Command_eoi___closed__5; return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3073_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3092_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; @@ -41814,7 +42129,7 @@ x_1 = l_Lean_Parser_Command_ctor___closed__8; return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__1() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -41824,7 +42139,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__2() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__2() { _start: { lean_object* x_1; @@ -41832,19 +42147,19 @@ x_1 = lean_mk_string_unchecked("declModifiersF", 14, 14); return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__3() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Parser_Term_quot___closed__1; x_2 = l_Lean_Parser_Term_quot___closed__2; x_3 = l_Lean_Parser_Command_quot___closed__1; -x_4 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__2; +x_4 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__2; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__4() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__4() { _start: { lean_object* x_1; lean_object* x_2; @@ -41854,7 +42169,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__5() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__5() { _start: { lean_object* x_1; lean_object* x_2; @@ -41864,7 +42179,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__6() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__6() { _start: { lean_object* x_1; lean_object* x_2; @@ -41874,12 +42189,12 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__7() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__7() { _start: { lean_object* x_1; lean_object* x_2; uint8_t x_3; lean_object* x_4; x_1 = lean_box(0); -x_2 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__6; +x_2 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__6; x_3 = 1; x_4 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_4, 0, x_1); @@ -41888,7 +42203,7 @@ lean_ctor_set_uint8(x_4, sizeof(void*)*2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__8() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__8() { _start: { lean_object* x_1; @@ -41896,17 +42211,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_declModifiersF_formatter) return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__9() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__9() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__8; +x_1 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__8; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__10() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__10() { _start: { lean_object* x_1; @@ -41914,7 +42229,7 @@ x_1 = l_Lean_PrettyPrinter_Formatter_formatterAliasesRef; return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__11() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__11() { _start: { lean_object* x_1; @@ -41922,17 +42237,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_declModifiersF_parenthesi return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__12() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__12() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__11; +x_1 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__11; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__13() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__13() { _start: { lean_object* x_1; @@ -41940,7 +42255,7 @@ x_1 = l_Lean_PrettyPrinter_Parenthesizer_parenthesizerAliasesRef; return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__14() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__14() { _start: { lean_object* x_1; @@ -41948,17 +42263,17 @@ x_1 = lean_mk_string_unchecked("nestedDeclModifiers", 19, 19); return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__15() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__14; +x_2 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__14; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__16() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__16() { _start: { lean_object* x_1; @@ -41966,19 +42281,19 @@ x_1 = lean_mk_string_unchecked("declModifiersT", 14, 14); return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__17() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__17() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Parser_Term_quot___closed__1; x_2 = l_Lean_Parser_Term_quot___closed__2; x_3 = l_Lean_Parser_Command_quot___closed__1; -x_4 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__16; +x_4 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__16; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__18() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__18() { _start: { lean_object* x_1; lean_object* x_2; @@ -41988,7 +42303,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__19() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__19() { _start: { lean_object* x_1; @@ -41996,17 +42311,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_declModifiersT_formatter) return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__20() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__20() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__19; +x_1 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__19; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__21() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__21() { _start: { lean_object* x_1; @@ -42014,17 +42329,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_declModifiersT_parenthesi return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__22() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__22() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__21; +x_1 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__21; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__23() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__23() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -42034,7 +42349,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__24() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__24() { _start: { lean_object* x_1; lean_object* x_2; @@ -42044,7 +42359,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__25() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__25() { _start: { lean_object* x_1; lean_object* x_2; @@ -42054,7 +42369,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__26() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__26() { _start: { lean_object* x_1; lean_object* x_2; @@ -42064,7 +42379,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__27() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__27() { _start: { lean_object* x_1; lean_object* x_2; @@ -42074,7 +42389,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__28() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__28() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -42084,7 +42399,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__29() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__29() { _start: { lean_object* x_1; lean_object* x_2; @@ -42094,7 +42409,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__30() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__30() { _start: { lean_object* x_1; lean_object* x_2; @@ -42104,7 +42419,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__31() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__31() { _start: { lean_object* x_1; lean_object* x_2; @@ -42114,7 +42429,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__32() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__32() { _start: { lean_object* x_1; lean_object* x_2; @@ -42124,7 +42439,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__33() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__33() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -42134,7 +42449,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__34() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__34() { _start: { lean_object* x_1; lean_object* x_2; @@ -42144,7 +42459,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__35() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__35() { _start: { lean_object* x_1; lean_object* x_2; @@ -42154,7 +42469,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__36() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__36() { _start: { lean_object* x_1; lean_object* x_2; @@ -42164,7 +42479,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__37() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__37() { _start: { lean_object* x_1; lean_object* x_2; @@ -42174,7 +42489,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__38() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__38() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -42184,7 +42499,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__39() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__39() { _start: { lean_object* x_1; lean_object* x_2; @@ -42194,7 +42509,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__40() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__40() { _start: { lean_object* x_1; lean_object* x_2; @@ -42204,7 +42519,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__41() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__41() { _start: { lean_object* x_1; lean_object* x_2; @@ -42214,7 +42529,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__42() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__42() { _start: { lean_object* x_1; lean_object* x_2; @@ -42224,7 +42539,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__43() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__43() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -42234,7 +42549,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__44() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__44() { _start: { lean_object* x_1; lean_object* x_2; @@ -42244,7 +42559,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__45() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__45() { _start: { lean_object* x_1; lean_object* x_2; @@ -42254,7 +42569,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__46() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__46() { _start: { lean_object* x_1; lean_object* x_2; @@ -42264,7 +42579,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__47() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__47() { _start: { lean_object* x_1; lean_object* x_2; @@ -42274,7 +42589,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__48() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__48() { _start: { lean_object* x_1; @@ -42282,29 +42597,29 @@ x_1 = lean_mk_string_unchecked("docComment", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__49() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__49() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__48; +x_2 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__48; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__50() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__50() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Parser_Term_quot___closed__1; x_2 = l_Lean_Parser_Term_quot___closed__2; x_3 = l_Lean_Parser_Command_quot___closed__1; -x_4 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__48; +x_4 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__48; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__51() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__51() { _start: { lean_object* x_1; lean_object* x_2; @@ -42314,17 +42629,17 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__52() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__52() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__50; +x_1 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__50; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__53() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__53() { _start: { lean_object* x_1; lean_object* x_2; @@ -42334,7 +42649,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__54() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__54() { _start: { lean_object* x_1; lean_object* x_2; @@ -42344,15 +42659,15 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_2 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__1; -x_3 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__3; -x_4 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__4; -x_5 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__5; -x_6 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__7; +x_2 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__1; +x_3 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__3; +x_4 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__4; +x_5 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__5; +x_6 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__7; x_7 = l_Lean_Parser_registerAlias(x_2, x_3, x_4, x_5, x_6, x_1); if (lean_obj_tag(x_7) == 0) { @@ -42360,8 +42675,8 @@ lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; x_8 = lean_ctor_get(x_7, 1); lean_inc(x_8); lean_dec(x_7); -x_9 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__10; -x_10 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__9; +x_9 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__10; +x_10 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__9; x_11 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_2, x_10, x_8); if (lean_obj_tag(x_11) == 0) { @@ -42369,8 +42684,8 @@ lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; x_12 = lean_ctor_get(x_11, 1); lean_inc(x_12); lean_dec(x_11); -x_13 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__13; -x_14 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__12; +x_13 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__13; +x_14 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__12; x_15 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_2, x_14, x_12); if (lean_obj_tag(x_15) == 0) { @@ -42378,9 +42693,9 @@ lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean x_16 = lean_ctor_get(x_15, 1); lean_inc(x_16); lean_dec(x_15); -x_17 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__15; -x_18 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__17; -x_19 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__18; +x_17 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__15; +x_18 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__17; +x_19 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__18; x_20 = l_Lean_Parser_registerAlias(x_17, x_18, x_19, x_5, x_6, x_16); if (lean_obj_tag(x_20) == 0) { @@ -42388,7 +42703,7 @@ lean_object* x_21; lean_object* x_22; lean_object* x_23; x_21 = lean_ctor_get(x_20, 1); lean_inc(x_21); lean_dec(x_20); -x_22 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__20; +x_22 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__20; x_23 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_17, x_22, x_21); if (lean_obj_tag(x_23) == 0) { @@ -42396,7 +42711,7 @@ lean_object* x_24; lean_object* x_25; lean_object* x_26; x_24 = lean_ctor_get(x_23, 1); lean_inc(x_24); lean_dec(x_23); -x_25 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__22; +x_25 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__22; x_26 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_17, x_25, x_24); if (lean_obj_tag(x_26) == 0) { @@ -42404,10 +42719,10 @@ lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean x_27 = lean_ctor_get(x_26, 1); lean_inc(x_27); lean_dec(x_26); -x_28 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__23; +x_28 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__23; x_29 = l_Lean_Parser_Command_declId___closed__2; -x_30 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__24; -x_31 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__25; +x_30 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__24; +x_31 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__25; x_32 = l_Lean_Parser_registerAlias(x_28, x_29, x_30, x_31, x_6, x_27); if (lean_obj_tag(x_32) == 0) { @@ -42415,7 +42730,7 @@ lean_object* x_33; lean_object* x_34; lean_object* x_35; x_33 = lean_ctor_get(x_32, 1); lean_inc(x_33); lean_dec(x_32); -x_34 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__26; +x_34 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__26; x_35 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_28, x_34, x_33); if (lean_obj_tag(x_35) == 0) { @@ -42423,7 +42738,7 @@ lean_object* x_36; lean_object* x_37; lean_object* x_38; x_36 = lean_ctor_get(x_35, 1); lean_inc(x_36); lean_dec(x_35); -x_37 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__27; +x_37 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__27; x_38 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_28, x_37, x_36); if (lean_obj_tag(x_38) == 0) { @@ -42431,10 +42746,10 @@ lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean x_39 = lean_ctor_get(x_38, 1); lean_inc(x_39); lean_dec(x_38); -x_40 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__28; +x_40 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__28; x_41 = l_Lean_Parser_Command_declSig___closed__2; -x_42 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__29; -x_43 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__30; +x_42 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__29; +x_43 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__30; x_44 = l_Lean_Parser_registerAlias(x_40, x_41, x_42, x_43, x_6, x_39); if (lean_obj_tag(x_44) == 0) { @@ -42442,7 +42757,7 @@ lean_object* x_45; lean_object* x_46; lean_object* x_47; x_45 = lean_ctor_get(x_44, 1); lean_inc(x_45); lean_dec(x_44); -x_46 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__31; +x_46 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__31; x_47 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_40, x_46, x_45); if (lean_obj_tag(x_47) == 0) { @@ -42450,7 +42765,7 @@ lean_object* x_48; lean_object* x_49; lean_object* x_50; x_48 = lean_ctor_get(x_47, 1); lean_inc(x_48); lean_dec(x_47); -x_49 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__32; +x_49 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__32; x_50 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_40, x_49, x_48); if (lean_obj_tag(x_50) == 0) { @@ -42458,10 +42773,10 @@ lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean x_51 = lean_ctor_get(x_50, 1); lean_inc(x_51); lean_dec(x_50); -x_52 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__33; +x_52 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__33; x_53 = l___regBuiltin_Lean_Parser_Command_declVal_docString__1___closed__2; -x_54 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__34; -x_55 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__35; +x_54 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__34; +x_55 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__35; x_56 = l_Lean_Parser_registerAlias(x_52, x_53, x_54, x_55, x_6, x_51); if (lean_obj_tag(x_56) == 0) { @@ -42469,7 +42784,7 @@ lean_object* x_57; lean_object* x_58; lean_object* x_59; x_57 = lean_ctor_get(x_56, 1); lean_inc(x_57); lean_dec(x_56); -x_58 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__36; +x_58 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__36; x_59 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_52, x_58, x_57); if (lean_obj_tag(x_59) == 0) { @@ -42477,7 +42792,7 @@ lean_object* x_60; lean_object* x_61; lean_object* x_62; x_60 = lean_ctor_get(x_59, 1); lean_inc(x_60); lean_dec(x_59); -x_61 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__37; +x_61 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__37; x_62 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_52, x_61, x_60); if (lean_obj_tag(x_62) == 0) { @@ -42485,10 +42800,10 @@ lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean x_63 = lean_ctor_get(x_62, 1); lean_inc(x_63); lean_dec(x_62); -x_64 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__38; +x_64 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__38; x_65 = l_Lean_Parser_Command_optDeclSig___closed__2; -x_66 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__39; -x_67 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__40; +x_66 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__39; +x_67 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__40; x_68 = l_Lean_Parser_registerAlias(x_64, x_65, x_66, x_67, x_6, x_63); if (lean_obj_tag(x_68) == 0) { @@ -42496,7 +42811,7 @@ lean_object* x_69; lean_object* x_70; lean_object* x_71; x_69 = lean_ctor_get(x_68, 1); lean_inc(x_69); lean_dec(x_68); -x_70 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__41; +x_70 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__41; x_71 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_64, x_70, x_69); if (lean_obj_tag(x_71) == 0) { @@ -42504,7 +42819,7 @@ lean_object* x_72; lean_object* x_73; lean_object* x_74; x_72 = lean_ctor_get(x_71, 1); lean_inc(x_72); lean_dec(x_71); -x_73 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__42; +x_73 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__42; x_74 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_64, x_73, x_72); if (lean_obj_tag(x_74) == 0) { @@ -42512,10 +42827,10 @@ lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean x_75 = lean_ctor_get(x_74, 1); lean_inc(x_75); lean_dec(x_74); -x_76 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__43; +x_76 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__43; x_77 = l___regBuiltin_Lean_Parser_Command_openDecl_docString__1___closed__2; -x_78 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__44; -x_79 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__45; +x_78 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__44; +x_79 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__45; x_80 = l_Lean_Parser_registerAlias(x_76, x_77, x_78, x_79, x_6, x_75); if (lean_obj_tag(x_80) == 0) { @@ -42523,7 +42838,7 @@ lean_object* x_81; lean_object* x_82; lean_object* x_83; x_81 = lean_ctor_get(x_80, 1); lean_inc(x_81); lean_dec(x_80); -x_82 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__46; +x_82 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__46; x_83 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_76, x_82, x_81); if (lean_obj_tag(x_83) == 0) { @@ -42531,7 +42846,7 @@ lean_object* x_84; lean_object* x_85; lean_object* x_86; x_84 = lean_ctor_get(x_83, 1); lean_inc(x_84); lean_dec(x_83); -x_85 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__47; +x_85 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__47; x_86 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_76, x_85, x_84); if (lean_obj_tag(x_86) == 0) { @@ -42539,10 +42854,10 @@ lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean x_87 = lean_ctor_get(x_86, 1); lean_inc(x_87); lean_dec(x_86); -x_88 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__49; -x_89 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__50; -x_90 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__51; -x_91 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__52; +x_88 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__49; +x_89 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__50; +x_90 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__51; +x_91 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__52; x_92 = l_Lean_Parser_registerAlias(x_88, x_89, x_90, x_91, x_6, x_87); if (lean_obj_tag(x_92) == 0) { @@ -42550,7 +42865,7 @@ lean_object* x_93; lean_object* x_94; lean_object* x_95; x_93 = lean_ctor_get(x_92, 1); lean_inc(x_93); lean_dec(x_92); -x_94 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__53; +x_94 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__53; x_95 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_88, x_94, x_93); if (lean_obj_tag(x_95) == 0) { @@ -42558,7 +42873,7 @@ lean_object* x_96; lean_object* x_97; lean_object* x_98; x_96 = lean_ctor_get(x_95, 1); lean_inc(x_96); lean_dec(x_95); -x_97 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__54; +x_97 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__54; x_98 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_88, x_97, x_96); return x_98; } @@ -49867,6 +50182,58 @@ lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_printTacTags_parenthesiz if (builtin) {res = l___regBuiltin_Lean_Parser_Command_printTacTags_parenthesizer__1(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +}l_Lean_Parser_Command_version___closed__1 = _init_l_Lean_Parser_Command_version___closed__1(); +lean_mark_persistent(l_Lean_Parser_Command_version___closed__1); +l_Lean_Parser_Command_version___closed__2 = _init_l_Lean_Parser_Command_version___closed__2(); +lean_mark_persistent(l_Lean_Parser_Command_version___closed__2); +l_Lean_Parser_Command_version___closed__3 = _init_l_Lean_Parser_Command_version___closed__3(); +lean_mark_persistent(l_Lean_Parser_Command_version___closed__3); +l_Lean_Parser_Command_version___closed__4 = _init_l_Lean_Parser_Command_version___closed__4(); +lean_mark_persistent(l_Lean_Parser_Command_version___closed__4); +l_Lean_Parser_Command_version___closed__5 = _init_l_Lean_Parser_Command_version___closed__5(); +lean_mark_persistent(l_Lean_Parser_Command_version___closed__5); +l_Lean_Parser_Command_version___closed__6 = _init_l_Lean_Parser_Command_version___closed__6(); +lean_mark_persistent(l_Lean_Parser_Command_version___closed__6); +l_Lean_Parser_Command_version___closed__7 = _init_l_Lean_Parser_Command_version___closed__7(); +lean_mark_persistent(l_Lean_Parser_Command_version___closed__7); +l_Lean_Parser_Command_version___closed__8 = _init_l_Lean_Parser_Command_version___closed__8(); +lean_mark_persistent(l_Lean_Parser_Command_version___closed__8); +l_Lean_Parser_Command_version = _init_l_Lean_Parser_Command_version(); +lean_mark_persistent(l_Lean_Parser_Command_version); +if (builtin) {res = l___regBuiltin_Lean_Parser_Command_version__1(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}l___regBuiltin_Lean_Parser_Command_version_docString__1___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_version_docString__1___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_version_docString__1___closed__1); +if (builtin) {res = l___regBuiltin_Lean_Parser_Command_version_docString__1(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}l_Lean_Parser_Command_version_formatter___closed__1 = _init_l_Lean_Parser_Command_version_formatter___closed__1(); +lean_mark_persistent(l_Lean_Parser_Command_version_formatter___closed__1); +l_Lean_Parser_Command_version_formatter___closed__2 = _init_l_Lean_Parser_Command_version_formatter___closed__2(); +lean_mark_persistent(l_Lean_Parser_Command_version_formatter___closed__2); +l_Lean_Parser_Command_version_formatter___closed__3 = _init_l_Lean_Parser_Command_version_formatter___closed__3(); +lean_mark_persistent(l_Lean_Parser_Command_version_formatter___closed__3); +l___regBuiltin_Lean_Parser_Command_version_formatter__1___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_version_formatter__1___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_version_formatter__1___closed__1); +l___regBuiltin_Lean_Parser_Command_version_formatter__1___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_version_formatter__1___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_version_formatter__1___closed__2); +if (builtin) {res = l___regBuiltin_Lean_Parser_Command_version_formatter__1(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}l_Lean_Parser_Command_version_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_version_parenthesizer___closed__1(); +lean_mark_persistent(l_Lean_Parser_Command_version_parenthesizer___closed__1); +l_Lean_Parser_Command_version_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_version_parenthesizer___closed__2(); +lean_mark_persistent(l_Lean_Parser_Command_version_parenthesizer___closed__2); +l_Lean_Parser_Command_version_parenthesizer___closed__3 = _init_l_Lean_Parser_Command_version_parenthesizer___closed__3(); +lean_mark_persistent(l_Lean_Parser_Command_version_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Command_version_parenthesizer__1___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_version_parenthesizer__1___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_version_parenthesizer__1___closed__1); +l___regBuiltin_Lean_Parser_Command_version_parenthesizer__1___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_version_parenthesizer__1___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_version_parenthesizer__1___closed__2); +if (builtin) {res = l___regBuiltin_Lean_Parser_Command_version_parenthesizer__1(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); }l_Lean_Parser_Command_init__quot___closed__1 = _init_l_Lean_Parser_Command_init__quot___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_init__quot___closed__1); l_Lean_Parser_Command_init__quot___closed__2 = _init_l_Lean_Parser_Command_init__quot___closed__2(); @@ -51713,122 +52080,122 @@ l_Lean_Parser_Command_eoi___closed__5 = _init_l_Lean_Parser_Command_eoi___closed lean_mark_persistent(l_Lean_Parser_Command_eoi___closed__5); l_Lean_Parser_Command_eoi = _init_l_Lean_Parser_Command_eoi(); lean_mark_persistent(l_Lean_Parser_Command_eoi); -if (builtin) {res = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3073_(lean_io_mk_world()); +if (builtin) {res = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3092_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l_Lean_Parser_Command_declModifiersF = _init_l_Lean_Parser_Command_declModifiersF(); lean_mark_persistent(l_Lean_Parser_Command_declModifiersF); l_Lean_Parser_Command_declModifiersT = _init_l_Lean_Parser_Command_declModifiersT(); lean_mark_persistent(l_Lean_Parser_Command_declModifiersT); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__1 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__1(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__1); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__2 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__2(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__2); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__3 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__3(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__3); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__4 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__4(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__4); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__5 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__5(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__5); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__6 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__6(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__6); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__7 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__7(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__7); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__8 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__8(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__8); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__9 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__9(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__9); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__10 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__10(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__10); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__11 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__11(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__11); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__12 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__12(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__12); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__13 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__13(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__13); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__14 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__14(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__14); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__15 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__15(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__15); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__16 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__16(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__16); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__17 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__17(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__17); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__18 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__18(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__18); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__19 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__19(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__19); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__20 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__20(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__20); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__21 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__21(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__21); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__22 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__22(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__22); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__23 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__23(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__23); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__24 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__24(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__24); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__25 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__25(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__25); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__26 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__26(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__26); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__27 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__27(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__27); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__28 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__28(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__28); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__29 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__29(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__29); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__30 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__30(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__30); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__31 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__31(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__31); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__32 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__32(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__32); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__33 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__33(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__33); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__34 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__34(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__34); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__35 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__35(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__35); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__36 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__36(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__36); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__37 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__37(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__37); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__38 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__38(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__38); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__39 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__39(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__39); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__40 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__40(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__40); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__41 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__41(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__41); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__42 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__42(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__42); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__43 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__43(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__43); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__44 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__44(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__44); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__45 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__45(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__45); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__46 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__46(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__46); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__47 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__47(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__47); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__48 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__48(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__48); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__49 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__49(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__49); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__50 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__50(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__50); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__51 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__51(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__51); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__52 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__52(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__52); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__53 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__53(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__53); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__54 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__54(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__54); -if (builtin) {res = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097_(lean_io_mk_world()); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__1 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__1(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__1); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__2 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__2(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__2); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__3 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__3(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__3); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__4 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__4(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__4); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__5 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__5(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__5); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__6 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__6(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__6); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__7 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__7(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__7); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__8 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__8(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__8); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__9 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__9(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__9); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__10 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__10(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__10); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__11 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__11(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__11); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__12 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__12(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__12); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__13 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__13(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__13); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__14 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__14(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__14); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__15 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__15(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__15); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__16 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__16(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__16); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__17 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__17(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__17); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__18 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__18(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__18); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__19 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__19(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__19); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__20 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__20(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__20); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__21 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__21(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__21); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__22 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__22(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__22); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__23 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__23(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__23); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__24 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__24(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__24); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__25 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__25(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__25); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__26 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__26(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__26); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__27 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__27(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__27); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__28 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__28(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__28); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__29 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__29(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__29); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__30 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__30(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__30); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__31 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__31(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__31); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__32 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__32(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__32); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__33 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__33(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__33); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__34 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__34(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__34); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__35 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__35(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__35); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__36 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__36(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__36); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__37 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__37(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__37); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__38 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__38(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__38); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__39 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__39(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__39); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__40 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__40(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__40); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__41 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__41(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__41); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__42 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__42(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__42); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__43 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__43(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__43); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__44 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__44(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__44); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__45 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__45(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__45); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__46 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__46(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__46); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__47 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__47(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__47); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__48 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__48(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__48); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__49 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__49(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__49); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__50 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__50(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__50); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__51 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__51(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__51); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__52 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__52(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__52); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__53 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__53(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__53); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__54 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__54(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__54); +if (builtin) {res = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l_Lean_Parser_Term_open___closed__1 = _init_l_Lean_Parser_Term_open___closed__1(); diff --git a/stage0/stdlib/Lean/Parser/Extra.c b/stage0/stdlib/Lean/Parser/Extra.c index 7b727c9e9a85..dd820afb91c8 100644 --- a/stage0/stdlib/Lean/Parser/Extra.c +++ b/stage0/stdlib/Lean/Parser/Extra.c @@ -19,12 +19,12 @@ LEAN_EXPORT lean_object* l_Lean_Parser_sepByIndent_parenthesizer___boxed(lean_ob LEAN_EXPORT lean_object* l_Lean_Parser_many1_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_Formatter_setLhsPrec_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ppHardSpace_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__20; lean_object* lean_string_utf8_extract(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__33; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__85; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__41; lean_object* l_Lean_Parser_checkColEq(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__63; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__86; LEAN_EXPORT lean_object* l_Lean_Parser_rawIdent_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_many_formatter___closed__3; lean_object* l_Lean_Syntax_mkNameLit(lean_object*, lean_object*); @@ -34,9 +34,11 @@ LEAN_EXPORT lean_object* l_Lean_Parser_identWithPartialTrailingDot; LEAN_EXPORT lean_object* l_Lean_Parser_ppHardLineUnlessUngrouped; LEAN_EXPORT lean_object* l_Lean_Parser_optional_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__37; +LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770_(lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_ppDedent_docString__1(lean_object*); static lean_object* l_Lean_Parser_sepByIndent_parenthesizer___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__5; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__65; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__17; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__57; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__19; static lean_object* l___regBuiltin_Lean_Parser_ppSpace_docString__1___closed__1; @@ -44,28 +46,27 @@ LEAN_EXPORT lean_object* l_Lean_Parser_ppHardSpace_parenthesizer(lean_object*, l extern lean_object* l_Lean_Parser_pushNone; LEAN_EXPORT lean_object* l_Lean_Parser_rawIdent_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__18; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__33; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__87; extern lean_object* l_Lean_Parser_nameLitNoAntiquot; static lean_object* l_Lean_Parser_identWithPartialTrailingDot_formatter___closed__6; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__53; lean_object* l_Lean_addBuiltinDocString(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_mkAntiquot_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_withCache_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ppRealGroup_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__81; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__26; LEAN_EXPORT lean_object* l_Lean_Parser_adaptCacheableContext_formatter(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_manyIndent_docString__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_ppRealGroup___boxed(lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__12; lean_object* l_Lean_PrettyPrinter_Formatter_orelse_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__48; static lean_object* l___regBuiltin_Lean_Parser_ppHardSpace_docString__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_withForbidden_parenthesizer___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__13; LEAN_EXPORT lean_object* l_Lean_ppLine_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_Formatter_fill(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__74; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__70; lean_object* l_Lean_PrettyPrinter_Formatter_rawIdentNoAntiquot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Parser_sepByIndent_formatter___spec__2___closed__4; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_ppHardSpace_docString__1(lean_object*); @@ -81,33 +82,35 @@ static lean_object* l___regBuiltin_Lean_Parser_strLit_docString__1___closed__1; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__50; uint8_t l_Lean_Exception_isInterrupt(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_charLit_docString__1___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__36; LEAN_EXPORT lean_object* l_Lean_Parser_ppRealFill___boxed(lean_object*); lean_object* l_Lean_TSyntax_getString(lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__34; static lean_object* l_Lean_Parser_charLit___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_withCache_formatter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__39; lean_object* l_Lean_PrettyPrinter_Formatter_checkPrec_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_identWithPartialTrailingDot___closed__8; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__38; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__11; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__75; static lean_object* l_Lean_ppDedent_formatter___closed__1; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__83; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__94; LEAN_EXPORT lean_object* l_Lean_Parser_many_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_charLit_docString__1(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__70; lean_object* l_Lean_Syntax_getId(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__77; LEAN_EXPORT lean_object* l_Lean_Parser_dbgTraceState_parenthesizer___boxed(lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Parser_sepByIndent_formatter___spec__2___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_ppGroup_docString__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_ppSpace_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_sepByIndent_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__43; static lean_object* l_Lean_Parser_strLit_formatter___closed__2; lean_object* lean_array_push(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_group_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_ident_docString__1(lean_object*); lean_object* l_Lean_PrettyPrinter_Formatter_sepByNoAntiquot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__57; static lean_object* l_Lean_Parser_mkAntiquot_parenthesizer___closed__5; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__57; LEAN_EXPORT lean_object* l_Lean_Parser_notSymbol(lean_object*); static lean_object* l_Lean_Parser_optional___closed__1; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__28; @@ -117,13 +120,15 @@ static lean_object* l_Lean_Parser_rawIdent___closed__1; static lean_object* l___regBuiltin_Lean_Parser_ppHardLineUnlessUngrouped_docString__1___closed__3; static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__8; static lean_object* l___regBuiltin_Lean_Parser_ppIndent_docString__1___closed__1; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__93; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__22; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__12; static lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_ppSpace_parenthesizer___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_sepBy1Indent_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__9; LEAN_EXPORT lean_object* l_Lean_Parser_notSymbol_parenthesizer___rarg(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__24; LEAN_EXPORT lean_object* l_Lean_Parser_evalInsideQuot_parenthesizer___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ppHardLineUnlessUngrouped_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter__1___closed__2; @@ -138,6 +143,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_dbgTraceState_formatter___rarg(lean_objec LEAN_EXPORT lean_object* l_Lean_Parser_optional(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_termParser_formatter___boxed(lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__61; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__37; LEAN_EXPORT lean_object* l_Lean_Parser_nameLit_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__25; static lean_object* l_Lean_Parser_strLit___closed__2; @@ -146,8 +152,9 @@ lean_object* lean_array_fget(lean_object*, lean_object*); lean_object* l_ReaderT_bind___at_Lean_PrettyPrinter_Formatter_categoryFormatterCore___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ppDedent_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29____________; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__38; LEAN_EXPORT lean_object* l_Lean_Parser_evalInsideQuot_parenthesizer___boxed(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__98; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__81; lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_mkAntiquotSplice_formatter___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_strLit; @@ -159,10 +166,10 @@ LEAN_EXPORT lean_object* l_Lean_Parser_withOpen_formatter(lean_object*, lean_obj lean_object* l_Lean_Parser_checkLinebreakBefore(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_withOpenDecl_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__30; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__88; lean_object* l_Lean_Macro_throwError___rarg(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__69; LEAN_EXPORT lean_object* l_Lean_Parser_withPositionAfterLinebreak_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__99; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__79; LEAN_EXPORT lean_object* l_Lean_Parser_incQuotDepth_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_scientificLit_parenthesizer___closed__1; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__18; @@ -173,15 +180,14 @@ static lean_object* l_Lean_Parser_mkAntiquot_parenthesizer___closed__8; lean_object* l_Lean_PrettyPrinter_Formatter_checkNoWsBefore_formatter___boxed(lean_object*); lean_object* l_Lean_Parser_orelse(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_ppDedentIfGrouped_docString__1___closed__2; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__7; lean_object* l_Lean_mkIdentFrom(lean_object*, lean_object*, uint8_t); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__23; static lean_object* l_Lean_Parser_mkAntiquotSplice_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_ppDedent_docString__1___closed__1; static lean_object* l_Lean_Parser_ident_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_decQuotDepth_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_hygieneInfo; lean_object* l_Lean_PrettyPrinter_Parenthesizer_checkColEq_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__52; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__14; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__55; static lean_object* l___regBuiltin_Lean_Parser_patternIgnore_docString__1___closed__2; @@ -191,6 +197,7 @@ lean_object* l_Lean_Syntax_node5(lean_object*, lean_object*, lean_object*, lean_ static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__4; static lean_object* l_Lean_Parser_antiquotExpr_formatter___closed__4; uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Parser_sepByIndent_formatter___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_withForbidden_formatter(lean_object*); static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__35; static lean_object* l_Lean_Parser_antiquotExpr_formatter___closed__3; @@ -199,12 +206,11 @@ static lean_object* l_Lean_Parser_group_formatter___closed__1; static lean_object* l_Lean_Parser_rawIdent_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_termParser_formatter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_scientificLit_formatter___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__86; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__91; LEAN_EXPORT lean_object* l_Lean_Parser_ppAllowUngrouped_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_nameLit_docString__1___closed__1; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__7; lean_object* l_Lean_PrettyPrinter_Formatter_tokenWithAntiquot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__21; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__30; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__56; static lean_object* l___regBuiltin_Lean_Parser_ppSpace_docString__1___closed__2; static lean_object* l_List_forIn_loop___at_Lean_Parser_sepByIndent_formatter___spec__2___closed__3; @@ -241,12 +247,11 @@ LEAN_EXPORT lean_object* l_Lean_Parser_sepByIndent_formatter___boxed(lean_object LEAN_EXPORT lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Parser_Basic_0__Lean_Parser_addQuotDepth_parenthesizer(lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__29; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__95; lean_object* l_Lean_PrettyPrinter_Parenthesizer_withAntiquotSuffixSplice_parenthesizer___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__6; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__97; LEAN_EXPORT lean_object* l_Lean_Parser_setExpected_formatter(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer__1___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__78; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__48; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_nameLit_docString__1(lean_object*); static lean_object* l_Lean_Parser_strLit_parenthesizer___closed__1; @@ -257,21 +262,23 @@ lean_object* l_Lean_PrettyPrinter_Formatter_withoutInfo_formatter(lean_object*, LEAN_EXPORT lean_object* l_Lean_Parser_setExpected_parenthesizer___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_sepByElemParser_formatter___closed__1; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__33; LEAN_EXPORT lean_object* l_Lean_Parser_mkAntiquot_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_ppDedentIfGrouped_docString__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ppAllowUngrouped_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_notSymbol_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__90; LEAN_EXPORT lean_object* l_Lean_Parser_ppGroup(lean_object*); size_t lean_usize_of_nat(lean_object*); lean_object* l_Lean_PrettyPrinter_Parenthesizer_checkNoWsBefore_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_identWithPartialTrailingDot_formatter___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_strLit_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_charLit_formatter___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__95; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__64; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__46; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__15; LEAN_EXPORT lean_object* l_Lean_Parser_notSymbol_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Macro_resolveGlobalName(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__58; static lean_object* l_Lean_Parser_antiquotExpr_parenthesizer___closed__3; static lean_object* l_Lean_Parser_many1Indent_formatter___closed__1; static lean_object* l_Lean_Parser_antiquotNestedExpr_formatter___closed__6; @@ -283,7 +290,6 @@ extern lean_object* l_Lean_Parser_hygieneInfoNoAntiquot; static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__14; static lean_object* l_Lean_Parser_scientificLit_formatter___closed__4; lean_object* l_Lean_Parser_optionalNoAntiquot(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__94; static lean_object* l_Lean_Parser_antiquotNestedExpr_formatter___closed__8; lean_object* lean_st_ref_take(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ident_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -292,17 +298,18 @@ static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Le static lean_object* l_Lean_ppHardSpace_formatter___closed__2; lean_object* l_Lean_Syntax_MonadTraverser_getCur___at_Lean_PrettyPrinter_Formatter_visitArgs___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__18; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__90; LEAN_EXPORT lean_object* l_Lean_Parser_setExpected_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_notSymbol_formatter___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_many1_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_commandParser_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__72; LEAN_EXPORT lean_object* l_Lean_Parser_commandParser_formatter(lean_object*); static lean_object* l_Lean_Parser_patternIgnore_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_withoutPosition_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_strLit___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__50; static lean_object* l_Lean_Parser_hygieneInfo_parenthesizer___closed__2; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__58; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__54; LEAN_EXPORT lean_object* l_Lean_Parser_ppRealFill_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Parser_charLitNoAntiquot; lean_object* l_Lean_SourceInfo_fromRef(lean_object*, uint8_t); @@ -315,21 +322,24 @@ static lean_object* l_Lean_Parser_identWithPartialTrailingDot_parenthesizer___cl LEAN_EXPORT lean_object* l_Lean_ppAllowUngrouped_formatter___boxed(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_ppHardLineUnlessUngrouped_docString__1___closed__2; lean_object* l_Lean_PrettyPrinter_Formatter_manyNoAntiquot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__87; LEAN_EXPORT lean_object* l_Lean_ppRealGroup_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__25; LEAN_EXPORT lean_object* l_Lean_Parser_sepByElemParser_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_ppLine_docString__1___closed__3; static lean_object* l___regBuiltin_Lean_Parser_numLit_docString__1___closed__3; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__62; LEAN_EXPORT lean_object* l_Lean_Parser_withOpen_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__9; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__61; lean_object* l_Lean_PrettyPrinter_Parenthesizer_checkColGe_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__69; static lean_object* l_Lean_Parser_identWithPartialTrailingDot_formatter___closed__1; lean_object* l_List_range(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_nonReservedSymbol_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__66; lean_object* l_Lean_PrettyPrinter_Parenthesizer_sepByNoAntiquot_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_Parenthesizer_atomic_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_antiquotNestedExpr_formatter___closed__4; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Parser_sepByIndent_formatter___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__78; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__23; static lean_object* l_Lean_Parser_charLit_formatter___closed__4; static lean_object* l___regBuiltin_Lean_Parser_charLit_docString__1___closed__2; @@ -337,32 +347,29 @@ static lean_object* l___regBuiltin_Lean_Parser_ppLine_docString__1___closed__1; extern lean_object* l_Lean_PrettyPrinter_parenthesizerAttribute; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__43; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter__1(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__73; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__14; LEAN_EXPORT lean_object* l_Lean_Parser_identWithPartialTrailingDot_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__52; static lean_object* l___regBuiltin_Lean_Parser_scientificLit_docString__1___closed__3; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__74; LEAN_EXPORT lean_object* l_Lean_Parser_numLit_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_mkAntiquot_parenthesizer___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_ppHardLineUnlessUngrouped_parenthesizer___rarg(lean_object*); extern lean_object* l_Lean_Parser_rawIdentNoAntiquot; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__59; static lean_object* l_Lean_Parser_sepByIndent_parenthesizer___closed__3; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__42; static lean_object* l_Lean_Parser_identWithPartialTrailingDot_parenthesizer___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__64; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__12; LEAN_EXPORT lean_object* l_Lean_Parser_adaptCacheableContext_formatter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_sepByElemParser_formatter___closed__3; LEAN_EXPORT lean_object* l_Lean_ppHardSpace_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__37; lean_object* l_Lean_quoteNameMk(lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__68; static lean_object* l_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__3; static lean_object* l_Lean_Parser_nameLit___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__31; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__40; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__96; static lean_object* l_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__4; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__32; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__44; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__9; lean_object* lean_st_ref_get(lean_object*, lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__54; @@ -372,7 +379,6 @@ static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Le LEAN_EXPORT lean_object* l_Lean_ppLine_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__46; lean_object* l_Lean_PrettyPrinter_Formatter_concat___lambda__1___boxed(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__65; static lean_object* l_Lean_Parser_nameLit_parenthesizer___closed__1; lean_object* l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_Formatter_nameLitNoAntiquot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -390,18 +396,16 @@ lean_object* l_Lean_Parser_notFollowedBy(lean_object*, lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__34; lean_object* l_Lean_PrettyPrinter_Formatter_pushWhitespace(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_identWithPartialTrailingDot_formatter___closed__7; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__1; lean_object* l_Lean_Parser_symbol(lean_object*); static lean_object* l_Lean_Parser_sepByIndent___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_sepBy1Indent_parenthesizer(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_withForbidden_parenthesizer___boxed(lean_object*); static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__25; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__37; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__74; static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_ppHardLineUnlessUngrouped_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Parser_sepByIndent_formatter___spec__3___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ppDedentIfGrouped_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__14; lean_object* l_Lean_Syntax_node3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_append(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ppGroup___boxed(lean_object*); @@ -411,6 +415,7 @@ static lean_object* l_Lean_Parser_commandParser_formatter___rarg___closed__2; static lean_object* l_Lean_Parser_mkAntiquotSplice_formatter___closed__2; static lean_object* l_Lean_Parser_nameLit___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_symbol_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__24; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__17; static lean_object* l___regBuiltin_Lean_Parser_ppRealGroup_docString__1___closed__3; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__40; @@ -418,30 +423,32 @@ LEAN_EXPORT lean_object* l_Lean_Parser_withResetCache_parenthesizer(lean_object* lean_object* l_Lean_PrettyPrinter_Parenthesizer_checkLinebreakBefore_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ppSpace; lean_object* l_Lean_PrettyPrinter_Formatter_optionalNoAntiquot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__8; static lean_object* l_Lean_Parser_optional_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_nameLit_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_scientificLit_docString__1___closed__2; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__97; LEAN_EXPORT lean_object* l_Lean_Parser_nameLit; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__19; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__8; static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__10; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__59; LEAN_EXPORT lean_object* l_Lean_Parser_suppressInsideQuot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__33; lean_object* l_Lean_Parser_checkNoWsBefore(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__92; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__3; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Parser_sepByIndent_formatter___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__5; static lean_object* l_Lean_Parser_sepByIndent___closed__2; static lean_object* l_Lean_Parser_hygieneInfo_formatter___closed__4; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__80; static lean_object* l_Lean_Parser_scientificLit___closed__1; static lean_object* l_Lean_Parser_mkAntiquot_parenthesizer___closed__9; static lean_object* l_Lean_Parser_strLit_formatter___closed__4; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Parser_sepByIndent_formatter___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__11; static lean_object* l_Lean_Parser_scientificLit_parenthesizer___closed__2; lean_object* l_Lean_Parser_withAntiquot(lean_object*, lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__23; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__13; static lean_object* l_Lean_Parser_sepByIndent___closed__3; lean_object* l_Lean_addMacroScope(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_Parenthesizer_withPosition_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -457,12 +464,11 @@ lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ppAllowUngrouped; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__6; static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__4; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__10; static lean_object* l_Lean_Parser_hygieneInfo_formatter___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__45; lean_object* l_Lean_PrettyPrinter_Parenthesizer_nonReservedSymbolNoAntiquot_parenthesizer___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_withForbidden_formatter___boxed(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__49; lean_object* l_Lean_Syntax_node2(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_ppHardSpace_docString__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_scientificLit_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -477,16 +483,17 @@ LEAN_EXPORT lean_object* l_Lean_Parser_withResetCache_formatter(lean_object*, le static lean_object* l_Lean_Parser_sepByElemParser_formatter___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Parser_Basic_0__Lean_Parser_addQuotDepth_parenthesizer___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_nonReservedSymbol_parenthesizer(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__80; lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__28; LEAN_EXPORT lean_object* l_Lean_Parser_withAntiquotSpliceAndSuffix_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__39; uint8_t l_Lean_Syntax_matchesNull(lean_object*, lean_object*); static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__11; static lean_object* l_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__2; static lean_object* l_Lean_Parser_nameLit_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_adaptCacheableContext_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer__1(lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__51; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__16; static lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter__1___closed__3; static lean_object* l_Lean_Parser_ident___closed__2; lean_object* l_Lean_Parser_many1NoAntiquot(lean_object*); @@ -510,9 +517,8 @@ static lean_object* l_Lean_Parser_identWithPartialTrailingDot___closed__4; static lean_object* l_Lean_Parser_charLit_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_ppRealFill_docString__1___closed__3; static lean_object* l_List_forIn_loop___at_Lean_Parser_sepByIndent_formatter___spec__2___closed__2; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__53; LEAN_EXPORT lean_object* l_Lean_Parser_ppHardSpace_parenthesizer___rarg(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__3; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Parser_sepByIndent_formatter___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_antiquotNestedExpr_formatter___closed__7; static lean_object* l_Lean_Parser_identWithPartialTrailingDot___closed__5; static lean_object* l___regBuiltin_Lean_Parser_ppGroup_docString__1___closed__2; @@ -521,19 +527,20 @@ static lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer_ static lean_object* l_Lean_Parser_rawIdent_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_commandParser_formatter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_withForbidden_formatter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__84; lean_object* l_Lean_Parser_andthen(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ppHardSpace; lean_object* l_Lean_PrettyPrinter_Parenthesizer_manyNoAntiquot_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_symbol_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__62; LEAN_EXPORT lean_object* l_Lean_Parser_withForbidden_parenthesizer(lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__29; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__20; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_strLit_docString__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_setExpected_parenthesizer___boxed(lean_object*); lean_object* l_Lean_Parser_checkColGe(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__62; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__44; static lean_object* l___regBuiltin_Lean_Parser_many1Indent_docString__1___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__88; static lean_object* l_Lean_Parser_charLit_formatter___closed__3; static lean_object* l_Lean_Parser_optional_formatter___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_evalInsideQuot_parenthesizer(lean_object*); @@ -542,7 +549,6 @@ LEAN_EXPORT lean_object* l_Lean_Parser_ppSpace_parenthesizer___boxed(lean_object static lean_object* l___regBuiltin_Lean_Parser_ppRealGroup_docString__1___closed__2; lean_object* lean_int_sub(lean_object*, lean_object*); static lean_object* l_Lean_Parser_numLit_formatter___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__32; LEAN_EXPORT lean_object* l_Lean_Parser_ident_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_charLit; LEAN_EXPORT lean_object* l_Lean_Parser_sepBy_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -554,7 +560,6 @@ static lean_object* l_Lean_Parser_termParser_formatter___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_rawIdent; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__2; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__8; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__26; LEAN_EXPORT lean_object* l_Lean_Parser_evalInsideQuot_formatter(lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__27; extern lean_object* l_Lean_PrettyPrinter_Formatter_formatterAliasesRef; @@ -564,62 +569,58 @@ LEAN_EXPORT lean_object* l_Lean_Parser_commandParser_formatter___boxed(lean_obje LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_hygieneInfo_docString__1(lean_object*); static lean_object* l_Lean_Parser_antiquotNestedExpr_formatter___closed__9; static lean_object* l_Lean_Parser_antiquotNestedExpr_formatter___closed__3; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__34; LEAN_EXPORT lean_object* l_Lean_Parser_sepByIndent_formatter___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Substring_takeWhileAux___at_Substring_trimLeft___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_scientificLit; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_many(lean_object*); LEAN_EXPORT lean_object* l_Lean_ppDedent_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_numLit_parenthesizer___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__43; lean_object* l_Lean_PrettyPrinter_Parenthesizer_unicodeSymbolNoAntiquot_parenthesizer___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__44; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__73; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__45; static lean_object* l_Lean_Parser_many1Indent___closed__1; static lean_object* l_Lean_Parser_hygieneInfo___closed__2; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__27; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__24; lean_object* l_Lean_PrettyPrinter_Formatter_pushNone_formatter___boxed(lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__51; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__16; LEAN_EXPORT lean_object* l_Lean_ppAllowUngrouped_formatter___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_many_formatter___closed__2; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__35; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__18; static lean_object* l___regBuiltin_Lean_Parser_numLit_docString__1___closed__2; static lean_object* l_Lean_Parser_antiquotNestedExpr_formatter___closed__2; static lean_object* l_Lean_Parser_scientificLit___closed__2; LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Parser_sepByIndent_formatter___spec__3(lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Parser_sepBy1Indent_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__67; static lean_object* l_Lean_Parser_mkAntiquot_parenthesizer___closed__1; static lean_object* l_Lean_Parser_mkAntiquotSplice_formatter___closed__4; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__45; LEAN_EXPORT lean_object* l_Lean_Parser_ppLine; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__91; LEAN_EXPORT lean_object* l_Lean_ppSpace_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_antiquotNestedExpr_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_ppIndent_docString__1___closed__3; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__27; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__55; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_manyIndent_docString__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_sepBy1Indent_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__11; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__32; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__42; static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__2; static lean_object* l_Lean_Parser_identWithPartialTrailingDot___closed__7; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__26; LEAN_EXPORT lean_object* l_Lean_Parser_withPosition_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_leadingNode_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_hygieneInfo_parenthesizer___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__56; lean_object* l_Lean_PrettyPrinter_Parenthesizer_withoutInfo_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_adaptCacheableContext_formatter___boxed(lean_object*); static lean_object* l_Lean_Parser_optional_formatter___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__29; LEAN_EXPORT lean_object* l___private_Lean_Parser_Basic_0__Lean_Parser_addQuotDepth_formatter___boxed(lean_object*); lean_object* l_Lean_Parser_registerAliasCore___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_patternIgnore_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_identWithPartialTrailingDot_parenthesizer___closed__4; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_termParser_formatter(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ident; LEAN_EXPORT lean_object* l_Lean_Parser_optional_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -634,26 +635,24 @@ lean_object* l_Lean_PrettyPrinter_Formatter_group(lean_object*, lean_object*, le static lean_object* l_Lean_Parser_scientificLit_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_manyIndent_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__53; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__12; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_many1Indent_docString__1(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__35; static lean_object* l___regBuiltin_Lean_Parser_ppDedent_docString__1___closed__3; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__93; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__82; static lean_object* l_Lean_Parser_strLit_formatter___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__71; static lean_object* l___regBuiltin_Lean_Parser_ppRealFill_docString__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_ppLine_parenthesizer___rarg(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__82; LEAN_EXPORT lean_object* l_Lean_Parser_withoutForbidden_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__55; lean_object* l_Lean_PrettyPrinter_Parenthesizer_scientificLitNoAntiquot_parenthesizer___boxed(lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__48; uint8_t lean_nat_dec_eq(lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_Formatter_visitArgs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__31; static lean_object* l_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__6; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__13; LEAN_EXPORT lean_object* l_Lean_Parser_ppAllowUngrouped_parenthesizer___rarg(lean_object*); lean_object* l_Lean_PrettyPrinter_Formatter_fold(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_dbgTraceState_formatter___boxed(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__96; static lean_object* l___regBuiltin_Lean_Parser_many_docString__1___closed__2; static lean_object* l___regBuiltin_Lean_Parser_many1_docString__1___closed__3; uint8_t lean_nat_dec_lt(lean_object*, lean_object*); @@ -662,17 +661,14 @@ lean_object* l_Substring_takeRightWhileAux___at_Substring_trimRight___spec__1(le LEAN_EXPORT lean_object* l_Lean_Parser_withCache_formatter___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_sepByElemParser_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_identWithPartialTrailingDot_parenthesizer___closed__6; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__17; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__2; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__39; LEAN_EXPORT lean_object* l_Lean_Parser_evalInsideQuot_formatter___boxed(lean_object*); lean_object* l_Lean_PrettyPrinter_Formatter_checkNoImmediateColon_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_atomic_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__22; static lean_object* l_Lean_Parser_ident_formatter___closed__3; lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ppGroup_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__10; static lean_object* l_Lean_Parser_identWithPartialTrailingDot_formatter___closed__4; extern lean_object* l_Lean_PrettyPrinter_Parenthesizer_parenthesizerAliasesRef; lean_object* l_Lean_Parser_withAntiquotSpliceAndSuffix(lean_object*, lean_object*, lean_object*); @@ -680,14 +676,12 @@ static lean_object* l_Lean_Parser_nameLit_formatter___closed__4; extern lean_object* l_Lean_Parser_skip; LEAN_EXPORT lean_object* l_Lean_Parser_decQuotDepth_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__24; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__18; static lean_object* l_Lean_Parser_charLit___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_ppIndent_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ppHardLineUnlessUngrouped_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_withoutPosition_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__16; extern lean_object* l_Lean_Parser_scientificLitNoAntiquot; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__72; LEAN_EXPORT lean_object* l_Lean_Parser_unicodeSymbol_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_identWithPartialTrailingDot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__13; @@ -696,6 +690,8 @@ lean_object* l_Lean_Syntax_node1(lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_ident_docString__1___closed__1; static lean_object* l_Lean_Parser_leadingNode_formatter___closed__2; lean_object* l_Lean_Parser_registerAlias(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__99; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__19; LEAN_EXPORT lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_group_docString__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_sepBy1Indent(lean_object*, lean_object*, lean_object*, uint8_t); @@ -712,10 +708,9 @@ LEAN_EXPORT lean_object* l_Lean_Parser_many1(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_nameLit_docString__1___closed__3; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__7; uint8_t l_Lean_Syntax_isNone(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__46; lean_object* l_Lean_PrettyPrinter_Formatter_withAntiquotSuffixSplice_formatter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__61; static lean_object* l_Lean_Parser_group_formatter___closed__2; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__84; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__20; static lean_object* l_Lean_Parser_strLit_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_manyIndent_docString__1___closed__2; @@ -724,6 +719,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_antiquotExpr_formatter(lean_object*, lean static lean_object* l_Lean_Parser_charLit_parenthesizer___closed__1; static lean_object* l_Lean_Parser_commandParser_formatter___rarg___closed__1; lean_object* lean_nat_sub(lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__63; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__21; lean_object* l_Std_Format_getIndent(lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__67; @@ -732,7 +728,6 @@ static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__13; static lean_object* l___regBuiltin_Lean_Parser_ppDedentIfGrouped_docString__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_mkAntiquotSplice_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_PrettyPrinter_backtrackExceptionId; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__40; LEAN_EXPORT lean_object* l_Lean_Parser_termParser_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Parser_Basic_0__Lean_Parser_addQuotDepth_formatter(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ppRealGroup(lean_object*); @@ -747,40 +742,42 @@ static lean_object* l_Lean_Parser_numLit_formatter___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_numLit_docString__1(lean_object*); extern lean_object* l_Lean_Parser_maxPrec; static lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter__1___closed__5; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__92; lean_object* l_Lean_Parser_sepBy(lean_object*, lean_object*, lean_object*, uint8_t); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__49; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__15; lean_object* l_Lean_PrettyPrinter_Formatter_strLitNoAntiquot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__52; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__21; extern lean_object* l_Lean_Parser_identNoAntiquot; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__66; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__60; static lean_object* l___regBuiltin_Lean_Parser_ppGroup_docString__1___closed__1; static lean_object* l_Lean_Parser_nameLit_parenthesizer___closed__2; lean_object* l_Lean_PrettyPrinter_Parenthesizer_charLitNoAntiquot_parenthesizer___boxed(lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__36; static lean_object* l_Lean_Parser_antiquotExpr_parenthesizer___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__54; lean_object* l_List_reverse___rarg(lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__30; LEAN_EXPORT lean_object* l_Lean_Parser_many1Indent_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__35; static lean_object* l_Lean_Parser_identWithPartialTrailingDot___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_mkAntiquotSplice_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__60; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_ppAllowUngrouped_docString__1(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__8; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__1; lean_object* l_String_intercalate(lean_object*, lean_object*); lean_object* lean_array_mk(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__51; static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__7; static lean_object* l___regBuiltin_Lean_Parser_ppSpace_docString__1___closed__3; static lean_object* l_Lean_Parser_identWithPartialTrailingDot___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_sepBy1_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_many1Indent_docString__1___closed__3; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__47; static lean_object* l___regBuiltin_Lean_Parser_ppIndent_docString__1___closed__2; lean_object* l_Lean_PrettyPrinter_Parenthesizer_tokenWithAntiquot_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_identWithPartialTrailingDot_parenthesizer___closed__5; static lean_object* l_Lean_Parser_identWithPartialTrailingDot_formatter___closed__3; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__26; size_t lean_usize_add(size_t, size_t); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__89; LEAN_EXPORT lean_object* l_Lean_Parser_sepByIndent(lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Parser_ppDedentIfGrouped(lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__6; @@ -794,11 +791,13 @@ static lean_object* l_Lean_Parser_many_formatter___closed__1; static lean_object* l_Lean_Parser_optional_formatter___closed__4; lean_object* lean_array_uget(lean_object*, size_t); LEAN_EXPORT lean_object* l_Lean_Parser_nodeWithAntiquot_formatter(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__56; static lean_object* l_Lean_Parser_numLit_formatter___closed__4; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__71; static lean_object* l___regBuiltin_Lean_Parser_ppHardSpace_docString__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_nodeWithAntiquot_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__28; LEAN_EXPORT lean_object* l_Lean_Parser_incQuotDepth_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__76; static lean_object* l_Lean_Parser_sepByIndent_formatter___closed__1; lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_ident_docString__1___closed__2; @@ -818,29 +817,33 @@ static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___ static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__47; static lean_object* l_Lean_Parser_optional_formatter___closed__2; lean_object* l_Lean_PrettyPrinter_Parenthesizer_rawIdentNoAntiquot_parenthesizer___boxed(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__27; LEAN_EXPORT lean_object* l_Lean_Parser_sepBy_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__15; static lean_object* l___regBuiltin_Lean_Parser_optional_docString__1___closed__2; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__30; static lean_object* l___regBuiltin_Lean_Parser_scientificLit_docString__1___closed__1; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__67; lean_object* lean_string_append(lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__31; LEAN_EXPORT lean_object* l_Lean_Parser_nonReservedSymbol_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_group_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_numLit_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Parser_Basic_0__Lean_Parser_addQuotDepth_formatter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_sepByIndent___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__16; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__50; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__49; lean_object* l_Lean_PrettyPrinter_Formatter_symbolNoAntiquot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_ppLine_docString__1(lean_object*); lean_object* lean_array_get_size(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_optional_docString__1___closed__1; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__6; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_many_docString__1(lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__47; static lean_object* l_Lean_Parser_mkAntiquotSplice_formatter___closed__3; static lean_object* l_Lean_Parser_numLit___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__60; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__42; static lean_object* l_Lean_Parser_mkAntiquot_parenthesizer___closed__3; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__98; static lean_object* l_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__5; lean_object* l_Lean_PrettyPrinter_Formatter_categoryParser_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_identWithPartialTrailingDot___closed__2; @@ -851,16 +854,15 @@ LEAN_EXPORT lean_object* l_Lean_Parser_sepBy1_parenthesizer(lean_object*, lean_o LEAN_EXPORT lean_object* l_Lean_Parser_notSymbol_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ppAllowUngrouped_formatter(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ppDedentIfGrouped_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__79; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__4; static lean_object* l_Lean_Parser_identWithPartialTrailingDot_formatter___closed__2; static lean_object* l_Lean_ppDedentIfGrouped_formatter___closed__1; lean_object* l_Lean_PrettyPrinter_Formatter_unicodeSymbolNoAntiquot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_evalInsideQuot_formatter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_mkAntiquotSplice_formatter___closed__6; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__75; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__73; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__31; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__68; uint8_t l_Lean_Exception_isRuntime(lean_object*); static lean_object* l_Lean_Parser_numLit_formatter___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_sepByIndent___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -873,10 +875,8 @@ static lean_object* l___regBuiltin_Lean_Parser_many1Indent_docString__1___closed static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__10; static lean_object* l_Lean_Parser_many1Indent_parenthesizer___closed__1; static lean_object* l_Lean_Parser_antiquotNestedExpr_formatter___closed__10; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__41; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__34; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__4; -LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789_(lean_object*); lean_object* l_String_toSubstring_x27(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_many_docString__1___closed__1; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__20; @@ -884,14 +884,18 @@ LEAN_EXPORT lean_object* l_Lean_Parser_withoutForbidden_parenthesizer(lean_objec static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__9; LEAN_EXPORT lean_object* l_Lean_Parser_dbgTraceState_formatter(lean_object*); static lean_object* l_Lean_Parser_sepByIndent___closed__5; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__76; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__1; static lean_object* l_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__1; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__25; lean_object* l_Lean_PrettyPrinter_Parenthesizer_hygieneInfoNoAntiquot_parenthesizer___boxed(lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__2; static lean_object* l_Lean_Parser_mkAntiquot_parenthesizer___closed__6; static lean_object* l___regBuiltin_Lean_Parser_manyIndent_docString__1___closed__1; static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__17; static lean_object* l_Lean_Parser_hygieneInfo_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_numLit_docString__1___closed__1; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__77; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_patternIgnore_docString__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ppDedentIfGrouped___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_adaptCacheableContext_parenthesizer___boxed(lean_object*); @@ -906,22 +910,18 @@ static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Le static lean_object* l_Lean_Parser_antiquotExpr_formatter___closed__1; static lean_object* l_Lean_Parser_antiquotNestedExpr_formatter___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_scientificLit_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__85; static lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter__1___closed__6; static lean_object* l___regBuiltin_Lean_Parser_ppRealGroup_docString__1___closed__1; static lean_object* l___regBuiltin_Lean_Parser_strLit_docString__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_ppGroup_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_Formatter_node_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__19; LEAN_EXPORT lean_object* l_Lean_Parser_nonReservedSymbol_formatter(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_identWithPartialTrailingDot_parenthesizer___closed__2; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__89; lean_object* l_Lean_PrettyPrinter_Parenthesizer_nameLitNoAntiquot_parenthesizer___boxed(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_strLit_docString__1___closed__3; static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__3; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__83; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__23; lean_object* l_Lean_PrettyPrinter_Parenthesizer_pushNone_parenthesizer___boxed(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__15; static lean_object* l_Lean_Parser_numLit_parenthesizer___closed__2; static lean_object* _init_l_Lean_Parser_leadingNode_formatter___closed__1() { _start: @@ -5012,88 +5012,86 @@ lean_dec(x_2); return x_6; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Parser_sepByIndent_formatter___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Parser_sepByIndent_formatter___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { -lean_object* x_8; uint8_t x_9; -x_8 = lean_unsigned_to_nat(0u); -x_9 = lean_nat_dec_eq(x_4, x_8); -if (x_9 == 0) -{ -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; lean_object* x_17; -x_10 = lean_unsigned_to_nat(1u); -x_11 = lean_nat_sub(x_4, x_10); -lean_dec(x_4); -x_12 = lean_array_fget(x_3, x_5); -x_13 = lean_array_get_size(x_2); -x_14 = lean_unsigned_to_nat(2u); -x_15 = lean_nat_mod(x_5, x_14); -x_16 = lean_nat_dec_eq(x_15, x_10); -lean_dec(x_15); -x_17 = lean_nat_add(x_5, x_10); -if (x_16 == 0) +lean_object* x_7; uint8_t x_8; +x_7 = lean_unsigned_to_nat(0u); +x_8 = lean_nat_dec_eq(x_3, x_7); +if (x_8 == 0) { -uint8_t x_18; lean_object* x_19; lean_object* x_20; +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; lean_object* x_15; +x_9 = lean_unsigned_to_nat(1u); +x_10 = lean_nat_sub(x_3, x_9); +lean_dec(x_3); +x_11 = lean_array_fget(x_2, x_4); +x_12 = lean_unsigned_to_nat(2u); +x_13 = lean_nat_mod(x_4, x_12); +x_14 = lean_nat_dec_eq(x_13, x_9); lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_5); -x_18 = 0; -x_19 = lean_box(x_18); -x_20 = lean_array_push(x_7, x_19); -x_4 = x_11; -x_5 = x_17; -x_6 = lean_box(0); -x_7 = x_20; +x_15 = lean_nat_add(x_4, x_9); +if (x_14 == 0) +{ +uint8_t x_16; lean_object* x_17; lean_object* x_18; +lean_dec(x_11); +lean_dec(x_4); +x_16 = 0; +x_17 = lean_box(x_16); +x_18 = lean_array_push(x_6, x_17); +x_3 = x_10; +x_4 = x_15; +x_5 = lean_box(0); +x_6 = x_18; goto _start; } else { -uint8_t x_22; -x_22 = l_Lean_Syntax_matchesNull(x_12, x_8); -if (x_22 == 0) +uint8_t x_20; +x_20 = l_Lean_Syntax_matchesNull(x_11, x_7); +if (x_20 == 0) { -uint8_t x_23; lean_object* x_24; lean_object* x_25; -lean_dec(x_13); -lean_dec(x_5); -x_23 = 0; -x_24 = lean_box(x_23); -x_25 = lean_array_push(x_7, x_24); -x_4 = x_11; -x_5 = x_17; -x_6 = lean_box(0); -x_7 = x_25; +uint8_t x_21; lean_object* x_22; lean_object* x_23; +lean_dec(x_4); +x_21 = 0; +x_22 = lean_box(x_21); +x_23 = lean_array_push(x_6, x_22); +x_3 = x_10; +x_4 = x_15; +x_5 = lean_box(0); +x_6 = x_23; goto _start; } else { -lean_object* x_27; uint8_t x_28; -x_27 = lean_nat_sub(x_13, x_10); -lean_dec(x_13); -x_28 = lean_nat_dec_eq(x_5, x_27); -lean_dec(x_27); -lean_dec(x_5); -if (x_28 == 0) -{ -uint8_t x_29; lean_object* x_30; lean_object* x_31; -x_29 = 1; -x_30 = lean_box(x_29); -x_31 = lean_array_push(x_7, x_30); -x_4 = x_11; -x_5 = x_17; -x_6 = lean_box(0); -x_7 = x_31; +lean_object* x_25; lean_object* x_26; uint8_t x_27; +x_25 = lean_array_get_size(x_1); +x_26 = lean_nat_sub(x_25, x_9); +lean_dec(x_25); +x_27 = lean_nat_dec_eq(x_4, x_26); +lean_dec(x_26); +lean_dec(x_4); +if (x_27 == 0) +{ +uint8_t x_28; lean_object* x_29; lean_object* x_30; +x_28 = 1; +x_29 = lean_box(x_28); +x_30 = lean_array_push(x_6, x_29); +x_3 = x_10; +x_4 = x_15; +x_5 = lean_box(0); +x_6 = x_30; goto _start; } else { -uint8_t x_33; lean_object* x_34; lean_object* x_35; -x_33 = 0; -x_34 = lean_box(x_33); -x_35 = lean_array_push(x_7, x_34); -x_4 = x_11; -x_5 = x_17; -x_6 = lean_box(0); -x_7 = x_35; +uint8_t x_32; lean_object* x_33; lean_object* x_34; +x_32 = 0; +x_33 = lean_box(x_32); +x_34 = lean_array_push(x_6, x_33); +x_3 = x_10; +x_4 = x_15; +x_5 = lean_box(0); +x_6 = x_34; goto _start; } } @@ -5101,9 +5099,9 @@ goto _start; } else { -lean_dec(x_5); lean_dec(x_4); -return x_7; +lean_dec(x_3); +return x_6; } } } @@ -5571,13 +5569,13 @@ x_11 = lean_ctor_get(x_9, 1); lean_inc(x_11); lean_dec(x_9); x_12 = l_Lean_Syntax_getArgs(x_10); +lean_dec(x_10); x_13 = lean_array_get_size(x_12); x_14 = lean_mk_empty_array_with_capacity(x_13); x_15 = lean_unsigned_to_nat(0u); lean_inc(x_13); -x_16 = l_Array_mapIdxM_map___at_Lean_Parser_sepByIndent_formatter___spec__1(x_10, x_12, x_12, x_13, x_15, lean_box(0), x_14); +x_16 = l_Array_mapFinIdxM_map___at_Lean_Parser_sepByIndent_formatter___spec__1(x_12, x_12, x_13, x_15, lean_box(0), x_14); lean_dec(x_12); -lean_dec(x_10); x_17 = lean_array_get_size(x_16); x_18 = lean_nat_dec_lt(x_15, x_17); lean_inc(x_13); @@ -5760,15 +5758,14 @@ return x_52; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Parser_sepByIndent_formatter___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Parser_sepByIndent_formatter___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { -lean_object* x_8; -x_8 = l_Array_mapIdxM_map___at_Lean_Parser_sepByIndent_formatter___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -lean_dec(x_3); +lean_object* x_7; +x_7 = l_Array_mapFinIdxM_map___at_Lean_Parser_sepByIndent_formatter___spec__1(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_2); lean_dec(x_1); -return x_8; +return x_7; } } LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Parser_sepByIndent_formatter___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { @@ -9387,7 +9384,7 @@ lean_dec(x_1); return x_6; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__1() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__1() { _start: { lean_object* x_1; @@ -9395,17 +9392,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_patternIgnore), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__2() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__1; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__1; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__3() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__3() { _start: { lean_object* x_1; lean_object* x_2; @@ -9415,7 +9412,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__4() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__4() { _start: { lean_object* x_1; lean_object* x_2; @@ -9425,12 +9422,12 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__5() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__5() { _start: { lean_object* x_1; lean_object* x_2; uint8_t x_3; lean_object* x_4; x_1 = lean_box(0); -x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__4; +x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__4; x_3 = 0; x_4 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_4, 0, x_1); @@ -9439,7 +9436,7 @@ lean_ctor_set_uint8(x_4, sizeof(void*)*2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__6() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__6() { _start: { lean_object* x_1; @@ -9447,17 +9444,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_patternIgnore_formatter), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__7() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__7() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__6; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__6; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__8() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__8() { _start: { lean_object* x_1; @@ -9465,7 +9462,7 @@ x_1 = l_Lean_PrettyPrinter_Formatter_formatterAliasesRef; return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__9() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__9() { _start: { lean_object* x_1; @@ -9473,17 +9470,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_patternIgnore_parenthesizer), 6, return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__10() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__10() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__9; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__9; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__11() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__11() { _start: { lean_object* x_1; @@ -9491,7 +9488,7 @@ x_1 = l_Lean_PrettyPrinter_Parenthesizer_parenthesizerAliasesRef; return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__12() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__12() { _start: { lean_object* x_1; @@ -9499,17 +9496,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_group), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__13() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__13() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__12; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__12; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__14() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__14() { _start: { lean_object* x_1; lean_object* x_2; @@ -9519,7 +9516,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__15() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__15() { _start: { lean_object* x_1; @@ -9527,17 +9524,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_group_formatter), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__16() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__16() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__15; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__15; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__17() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__17() { _start: { lean_object* x_1; @@ -9545,17 +9542,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_group_parenthesizer), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__18() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__18() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__17; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__17; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__19() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__19() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -9565,7 +9562,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__20() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__20() { _start: { lean_object* x_1; lean_object* x_2; @@ -9575,7 +9572,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__21() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__21() { _start: { lean_object* x_1; lean_object* x_2; @@ -9585,7 +9582,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__22() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__22() { _start: { lean_object* x_1; lean_object* x_2; @@ -9595,12 +9592,12 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__23() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__23() { _start: { lean_object* x_1; lean_object* x_2; uint8_t x_3; lean_object* x_4; x_1 = lean_box(0); -x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__22; +x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__22; x_3 = 1; x_4 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_4, 0, x_1); @@ -9609,7 +9606,7 @@ lean_ctor_set_uint8(x_4, sizeof(void*)*2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__24() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__24() { _start: { lean_object* x_1; @@ -9617,17 +9614,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_ppHardSpace_formatter___boxed), 5, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__25() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__25() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__24; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__24; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__26() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__26() { _start: { lean_object* x_1; @@ -9635,17 +9632,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppHardSpace_parenthesizer___boxed return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__27() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__27() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__26; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__26; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__28() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__28() { _start: { lean_object* x_1; lean_object* x_2; @@ -9655,7 +9652,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__29() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__29() { _start: { lean_object* x_1; @@ -9663,17 +9660,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_ppSpace_formatter___boxed), 5, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__30() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__30() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__29; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__29; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__31() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__31() { _start: { lean_object* x_1; @@ -9681,17 +9678,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppSpace_parenthesizer___boxed), 4 return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__32() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__32() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__31; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__31; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__33() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__33() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -9701,7 +9698,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__34() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__34() { _start: { lean_object* x_1; lean_object* x_2; @@ -9711,7 +9708,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__35() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__35() { _start: { lean_object* x_1; @@ -9719,17 +9716,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_ppLine_formatter___boxed), 5, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__36() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__36() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__35; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__35; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__37() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__37() { _start: { lean_object* x_1; @@ -9737,17 +9734,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppLine_parenthesizer___boxed), 4, return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__38() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__38() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__37; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__37; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__39() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__39() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -9757,7 +9754,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__40() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__40() { _start: { lean_object* x_1; @@ -9765,17 +9762,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppGroup___boxed), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__41() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__41() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__40; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__40; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__42() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__42() { _start: { lean_object* x_1; lean_object* x_2; @@ -9785,7 +9782,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__43() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__43() { _start: { lean_object* x_1; lean_object* x_2; uint8_t x_3; lean_object* x_4; @@ -9799,7 +9796,7 @@ lean_ctor_set_uint8(x_4, sizeof(void*)*2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__44() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__44() { _start: { lean_object* x_1; @@ -9807,17 +9804,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppGroup_formatter), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__45() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__45() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__44; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__44; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__46() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__46() { _start: { lean_object* x_1; @@ -9825,17 +9822,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppGroup_parenthesizer), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__47() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__47() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__46; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__46; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__48() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__48() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -9845,7 +9842,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__49() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__49() { _start: { lean_object* x_1; @@ -9853,17 +9850,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppRealGroup___boxed), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__50() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__50() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__49; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__49; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__51() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__51() { _start: { lean_object* x_1; lean_object* x_2; @@ -9873,7 +9870,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__52() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__52() { _start: { lean_object* x_1; @@ -9881,17 +9878,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_ppRealGroup_formatter), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__53() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__53() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__52; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__52; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__54() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__54() { _start: { lean_object* x_1; @@ -9899,17 +9896,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppRealGroup_parenthesizer), 6, 0) return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__55() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__55() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__54; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__54; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__56() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__56() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -9919,7 +9916,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__57() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__57() { _start: { lean_object* x_1; @@ -9927,17 +9924,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppRealFill___boxed), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__58() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__58() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__57; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__57; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__59() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__59() { _start: { lean_object* x_1; lean_object* x_2; @@ -9947,7 +9944,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__60() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__60() { _start: { lean_object* x_1; @@ -9955,17 +9952,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_ppRealFill_formatter), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__61() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__61() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__60; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__60; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__62() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__62() { _start: { lean_object* x_1; @@ -9973,17 +9970,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppRealFill_parenthesizer), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__63() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__63() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__62; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__62; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__64() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__64() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -9993,7 +9990,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__65() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__65() { _start: { lean_object* x_1; @@ -10001,17 +9998,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppIndent___boxed), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__66() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__66() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__65; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__65; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__67() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__67() { _start: { lean_object* x_1; lean_object* x_2; @@ -10021,7 +10018,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__68() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__68() { _start: { lean_object* x_1; @@ -10029,17 +10026,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_ppIndent_formatter), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__69() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__69() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__68; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__68; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__70() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__70() { _start: { lean_object* x_1; @@ -10047,17 +10044,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppIndent_parenthesizer), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__71() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__71() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__70; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__70; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__72() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__72() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -10067,7 +10064,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__73() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__73() { _start: { lean_object* x_1; @@ -10075,17 +10072,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppDedent___boxed), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__74() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__74() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__73; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__73; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__75() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__75() { _start: { lean_object* x_1; lean_object* x_2; @@ -10095,7 +10092,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__76() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__76() { _start: { lean_object* x_1; @@ -10103,17 +10100,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_ppDedent_formatter), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__77() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__77() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__76; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__76; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__78() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__78() { _start: { lean_object* x_1; @@ -10121,17 +10118,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppDedent_parenthesizer), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__79() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__79() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__78; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__78; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__80() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__80() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -10141,7 +10138,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__81() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__81() { _start: { lean_object* x_1; @@ -10149,17 +10146,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppDedentIfGrouped___boxed), 1, 0) return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__82() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__82() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__81; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__81; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__83() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__83() { _start: { lean_object* x_1; lean_object* x_2; @@ -10169,7 +10166,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__84() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__84() { _start: { lean_object* x_1; @@ -10177,17 +10174,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_ppDedentIfGrouped_formatter), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__85() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__85() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__84; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__84; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__86() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__86() { _start: { lean_object* x_1; @@ -10195,17 +10192,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppDedentIfGrouped_parenthesizer), return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__87() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__87() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__86; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__86; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__88() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__88() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -10215,7 +10212,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__89() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__89() { _start: { lean_object* x_1; lean_object* x_2; @@ -10225,7 +10222,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__90() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__90() { _start: { lean_object* x_1; @@ -10233,17 +10230,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_ppAllowUngrouped_formatter___boxed), 1, return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__91() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__91() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__90; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__90; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__92() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__92() { _start: { lean_object* x_1; @@ -10251,17 +10248,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppAllowUngrouped_parenthesizer___ return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__93() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__93() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__92; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__92; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__94() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__94() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -10271,7 +10268,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__95() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__95() { _start: { lean_object* x_1; lean_object* x_2; @@ -10281,7 +10278,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__96() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__96() { _start: { lean_object* x_1; @@ -10289,17 +10286,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_ppHardLineUnlessUngrouped_formatter___bo return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__97() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__97() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__96; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__96; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__98() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__98() { _start: { lean_object* x_1; @@ -10307,25 +10304,25 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppHardLineUnlessUngrouped_parenth return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__99() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__99() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__98; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__98; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_2 = l_Lean_Parser_patternIgnore_formatter___closed__2; x_3 = l___regBuiltin_Lean_Parser_patternIgnore_docString__1___closed__1; -x_4 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__2; -x_5 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__3; -x_6 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__5; +x_4 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__2; +x_5 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__3; +x_6 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__5; x_7 = l_Lean_Parser_registerAlias(x_2, x_3, x_4, x_5, x_6, x_1); if (lean_obj_tag(x_7) == 0) { @@ -10333,8 +10330,8 @@ lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; x_8 = lean_ctor_get(x_7, 1); lean_inc(x_8); lean_dec(x_7); -x_9 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__8; -x_10 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__7; +x_9 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__8; +x_10 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__7; x_11 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_2, x_10, x_8); if (lean_obj_tag(x_11) == 0) { @@ -10342,8 +10339,8 @@ lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; x_12 = lean_ctor_get(x_11, 1); lean_inc(x_12); lean_dec(x_11); -x_13 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__11; -x_14 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__10; +x_13 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__11; +x_14 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__10; x_15 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_2, x_14, x_12); if (lean_obj_tag(x_15) == 0) { @@ -10353,8 +10350,8 @@ lean_inc(x_16); lean_dec(x_15); x_17 = l_Lean_Parser_group_formatter___closed__2; x_18 = l___regBuiltin_Lean_Parser_group_docString__1___closed__1; -x_19 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__13; -x_20 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__14; +x_19 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__13; +x_20 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__14; x_21 = l_Lean_Parser_registerAlias(x_17, x_18, x_19, x_20, x_6, x_16); if (lean_obj_tag(x_21) == 0) { @@ -10362,7 +10359,7 @@ lean_object* x_22; lean_object* x_23; lean_object* x_24; x_22 = lean_ctor_get(x_21, 1); lean_inc(x_22); lean_dec(x_21); -x_23 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__16; +x_23 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__16; x_24 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_17, x_23, x_22); if (lean_obj_tag(x_24) == 0) { @@ -10370,7 +10367,7 @@ lean_object* x_25; lean_object* x_26; lean_object* x_27; x_25 = lean_ctor_get(x_24, 1); lean_inc(x_25); lean_dec(x_24); -x_26 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__18; +x_26 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__18; x_27 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_17, x_26, x_25); if (lean_obj_tag(x_27) == 0) { @@ -10378,11 +10375,11 @@ lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean x_28 = lean_ctor_get(x_27, 1); lean_inc(x_28); lean_dec(x_27); -x_29 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__19; +x_29 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__19; x_30 = l___regBuiltin_Lean_Parser_ppHardSpace_docString__1___closed__2; -x_31 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__20; -x_32 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__21; -x_33 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__23; +x_31 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__20; +x_32 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__21; +x_33 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__23; x_34 = l_Lean_Parser_registerAlias(x_29, x_30, x_31, x_32, x_33, x_28); if (lean_obj_tag(x_34) == 0) { @@ -10390,7 +10387,7 @@ lean_object* x_35; lean_object* x_36; lean_object* x_37; x_35 = lean_ctor_get(x_34, 1); lean_inc(x_35); lean_dec(x_34); -x_36 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__25; +x_36 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__25; x_37 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_29, x_36, x_35); if (lean_obj_tag(x_37) == 0) { @@ -10398,7 +10395,7 @@ lean_object* x_38; lean_object* x_39; lean_object* x_40; x_38 = lean_ctor_get(x_37, 1); lean_inc(x_38); lean_dec(x_37); -x_39 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__27; +x_39 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__27; x_40 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_29, x_39, x_38); if (lean_obj_tag(x_40) == 0) { @@ -10408,7 +10405,7 @@ lean_inc(x_41); lean_dec(x_40); x_42 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__23; x_43 = l___regBuiltin_Lean_Parser_ppSpace_docString__1___closed__2; -x_44 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__28; +x_44 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__28; x_45 = l_Lean_Parser_registerAlias(x_42, x_43, x_31, x_44, x_33, x_41); if (lean_obj_tag(x_45) == 0) { @@ -10416,7 +10413,7 @@ lean_object* x_46; lean_object* x_47; lean_object* x_48; x_46 = lean_ctor_get(x_45, 1); lean_inc(x_46); lean_dec(x_45); -x_47 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__30; +x_47 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__30; x_48 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_42, x_47, x_46); if (lean_obj_tag(x_48) == 0) { @@ -10424,7 +10421,7 @@ lean_object* x_49; lean_object* x_50; lean_object* x_51; x_49 = lean_ctor_get(x_48, 1); lean_inc(x_49); lean_dec(x_48); -x_50 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__32; +x_50 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__32; x_51 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_42, x_50, x_49); if (lean_obj_tag(x_51) == 0) { @@ -10432,9 +10429,9 @@ lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean x_52 = lean_ctor_get(x_51, 1); lean_inc(x_52); lean_dec(x_51); -x_53 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__33; +x_53 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__33; x_54 = l___regBuiltin_Lean_Parser_ppLine_docString__1___closed__2; -x_55 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__34; +x_55 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__34; x_56 = l_Lean_Parser_registerAlias(x_53, x_54, x_31, x_55, x_33, x_52); if (lean_obj_tag(x_56) == 0) { @@ -10442,7 +10439,7 @@ lean_object* x_57; lean_object* x_58; lean_object* x_59; x_57 = lean_ctor_get(x_56, 1); lean_inc(x_57); lean_dec(x_56); -x_58 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__36; +x_58 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__36; x_59 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_53, x_58, x_57); if (lean_obj_tag(x_59) == 0) { @@ -10450,7 +10447,7 @@ lean_object* x_60; lean_object* x_61; lean_object* x_62; x_60 = lean_ctor_get(x_59, 1); lean_inc(x_60); lean_dec(x_59); -x_61 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__38; +x_61 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__38; x_62 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_53, x_61, x_60); if (lean_obj_tag(x_62) == 0) { @@ -10458,11 +10455,11 @@ lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean x_63 = lean_ctor_get(x_62, 1); lean_inc(x_63); lean_dec(x_62); -x_64 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__39; +x_64 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__39; x_65 = l___regBuiltin_Lean_Parser_ppGroup_docString__1___closed__2; -x_66 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__41; -x_67 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__42; -x_68 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__43; +x_66 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__41; +x_67 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__42; +x_68 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__43; x_69 = l_Lean_Parser_registerAlias(x_64, x_65, x_66, x_67, x_68, x_63); if (lean_obj_tag(x_69) == 0) { @@ -10470,7 +10467,7 @@ lean_object* x_70; lean_object* x_71; lean_object* x_72; x_70 = lean_ctor_get(x_69, 1); lean_inc(x_70); lean_dec(x_69); -x_71 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__45; +x_71 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__45; x_72 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_64, x_71, x_70); if (lean_obj_tag(x_72) == 0) { @@ -10478,7 +10475,7 @@ lean_object* x_73; lean_object* x_74; lean_object* x_75; x_73 = lean_ctor_get(x_72, 1); lean_inc(x_73); lean_dec(x_72); -x_74 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__47; +x_74 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__47; x_75 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_64, x_74, x_73); if (lean_obj_tag(x_75) == 0) { @@ -10486,10 +10483,10 @@ lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean x_76 = lean_ctor_get(x_75, 1); lean_inc(x_76); lean_dec(x_75); -x_77 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__48; +x_77 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__48; x_78 = l___regBuiltin_Lean_Parser_ppRealGroup_docString__1___closed__2; -x_79 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__50; -x_80 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__51; +x_79 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__50; +x_80 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__51; x_81 = l_Lean_Parser_registerAlias(x_77, x_78, x_79, x_80, x_68, x_76); if (lean_obj_tag(x_81) == 0) { @@ -10497,7 +10494,7 @@ lean_object* x_82; lean_object* x_83; lean_object* x_84; x_82 = lean_ctor_get(x_81, 1); lean_inc(x_82); lean_dec(x_81); -x_83 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__53; +x_83 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__53; x_84 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_77, x_83, x_82); if (lean_obj_tag(x_84) == 0) { @@ -10505,7 +10502,7 @@ lean_object* x_85; lean_object* x_86; lean_object* x_87; x_85 = lean_ctor_get(x_84, 1); lean_inc(x_85); lean_dec(x_84); -x_86 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__55; +x_86 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__55; x_87 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_77, x_86, x_85); if (lean_obj_tag(x_87) == 0) { @@ -10513,10 +10510,10 @@ lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean x_88 = lean_ctor_get(x_87, 1); lean_inc(x_88); lean_dec(x_87); -x_89 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__56; +x_89 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__56; x_90 = l___regBuiltin_Lean_Parser_ppRealFill_docString__1___closed__2; -x_91 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__58; -x_92 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__59; +x_91 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__58; +x_92 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__59; x_93 = l_Lean_Parser_registerAlias(x_89, x_90, x_91, x_92, x_68, x_88); if (lean_obj_tag(x_93) == 0) { @@ -10524,7 +10521,7 @@ lean_object* x_94; lean_object* x_95; lean_object* x_96; x_94 = lean_ctor_get(x_93, 1); lean_inc(x_94); lean_dec(x_93); -x_95 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__61; +x_95 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__61; x_96 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_89, x_95, x_94); if (lean_obj_tag(x_96) == 0) { @@ -10532,7 +10529,7 @@ lean_object* x_97; lean_object* x_98; lean_object* x_99; x_97 = lean_ctor_get(x_96, 1); lean_inc(x_97); lean_dec(x_96); -x_98 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__63; +x_98 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__63; x_99 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_89, x_98, x_97); if (lean_obj_tag(x_99) == 0) { @@ -10540,10 +10537,10 @@ lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; x_100 = lean_ctor_get(x_99, 1); lean_inc(x_100); lean_dec(x_99); -x_101 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__64; +x_101 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__64; x_102 = l___regBuiltin_Lean_Parser_ppIndent_docString__1___closed__2; -x_103 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__66; -x_104 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__67; +x_103 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__66; +x_104 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__67; x_105 = l_Lean_Parser_registerAlias(x_101, x_102, x_103, x_104, x_68, x_100); if (lean_obj_tag(x_105) == 0) { @@ -10551,7 +10548,7 @@ lean_object* x_106; lean_object* x_107; lean_object* x_108; x_106 = lean_ctor_get(x_105, 1); lean_inc(x_106); lean_dec(x_105); -x_107 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__69; +x_107 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__69; x_108 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_101, x_107, x_106); if (lean_obj_tag(x_108) == 0) { @@ -10559,7 +10556,7 @@ lean_object* x_109; lean_object* x_110; lean_object* x_111; x_109 = lean_ctor_get(x_108, 1); lean_inc(x_109); lean_dec(x_108); -x_110 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__71; +x_110 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__71; x_111 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_101, x_110, x_109); if (lean_obj_tag(x_111) == 0) { @@ -10567,10 +10564,10 @@ lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; x_112 = lean_ctor_get(x_111, 1); lean_inc(x_112); lean_dec(x_111); -x_113 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__72; +x_113 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__72; x_114 = l___regBuiltin_Lean_Parser_ppDedent_docString__1___closed__2; -x_115 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__74; -x_116 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__75; +x_115 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__74; +x_116 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__75; x_117 = l_Lean_Parser_registerAlias(x_113, x_114, x_115, x_116, x_68, x_112); if (lean_obj_tag(x_117) == 0) { @@ -10578,7 +10575,7 @@ lean_object* x_118; lean_object* x_119; lean_object* x_120; x_118 = lean_ctor_get(x_117, 1); lean_inc(x_118); lean_dec(x_117); -x_119 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__77; +x_119 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__77; x_120 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_113, x_119, x_118); if (lean_obj_tag(x_120) == 0) { @@ -10586,7 +10583,7 @@ lean_object* x_121; lean_object* x_122; lean_object* x_123; x_121 = lean_ctor_get(x_120, 1); lean_inc(x_121); lean_dec(x_120); -x_122 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__79; +x_122 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__79; x_123 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_113, x_122, x_121); if (lean_obj_tag(x_123) == 0) { @@ -10594,10 +10591,10 @@ lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; x_124 = lean_ctor_get(x_123, 1); lean_inc(x_124); lean_dec(x_123); -x_125 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__80; +x_125 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__80; x_126 = l___regBuiltin_Lean_Parser_ppDedentIfGrouped_docString__1___closed__2; -x_127 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__82; -x_128 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__83; +x_127 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__82; +x_128 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__83; x_129 = l_Lean_Parser_registerAlias(x_125, x_126, x_127, x_128, x_68, x_124); if (lean_obj_tag(x_129) == 0) { @@ -10605,7 +10602,7 @@ lean_object* x_130; lean_object* x_131; lean_object* x_132; x_130 = lean_ctor_get(x_129, 1); lean_inc(x_130); lean_dec(x_129); -x_131 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__85; +x_131 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__85; x_132 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_125, x_131, x_130); if (lean_obj_tag(x_132) == 0) { @@ -10613,7 +10610,7 @@ lean_object* x_133; lean_object* x_134; lean_object* x_135; x_133 = lean_ctor_get(x_132, 1); lean_inc(x_133); lean_dec(x_132); -x_134 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__87; +x_134 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__87; x_135 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_125, x_134, x_133); if (lean_obj_tag(x_135) == 0) { @@ -10621,9 +10618,9 @@ lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; x_136 = lean_ctor_get(x_135, 1); lean_inc(x_136); lean_dec(x_135); -x_137 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__88; +x_137 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__88; x_138 = l___regBuiltin_Lean_Parser_ppAllowUngrouped_docString__1___closed__2; -x_139 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__89; +x_139 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__89; x_140 = l_Lean_Parser_registerAlias(x_137, x_138, x_31, x_139, x_33, x_136); if (lean_obj_tag(x_140) == 0) { @@ -10631,7 +10628,7 @@ lean_object* x_141; lean_object* x_142; lean_object* x_143; x_141 = lean_ctor_get(x_140, 1); lean_inc(x_141); lean_dec(x_140); -x_142 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__91; +x_142 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__91; x_143 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_137, x_142, x_141); if (lean_obj_tag(x_143) == 0) { @@ -10639,7 +10636,7 @@ lean_object* x_144; lean_object* x_145; lean_object* x_146; x_144 = lean_ctor_get(x_143, 1); lean_inc(x_144); lean_dec(x_143); -x_145 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__93; +x_145 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__93; x_146 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_137, x_145, x_144); if (lean_obj_tag(x_146) == 0) { @@ -10647,9 +10644,9 @@ lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; x_147 = lean_ctor_get(x_146, 1); lean_inc(x_147); lean_dec(x_146); -x_148 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__94; +x_148 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__94; x_149 = l___regBuiltin_Lean_Parser_ppHardLineUnlessUngrouped_docString__1___closed__2; -x_150 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__95; +x_150 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__95; x_151 = l_Lean_Parser_registerAlias(x_148, x_149, x_31, x_150, x_33, x_147); if (lean_obj_tag(x_151) == 0) { @@ -10657,7 +10654,7 @@ lean_object* x_152; lean_object* x_153; lean_object* x_154; x_152 = lean_ctor_get(x_151, 1); lean_inc(x_152); lean_dec(x_151); -x_153 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__97; +x_153 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__97; x_154 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_148, x_153, x_152); if (lean_obj_tag(x_154) == 0) { @@ -10665,7 +10662,7 @@ lean_object* x_155; lean_object* x_156; lean_object* x_157; x_155 = lean_ctor_get(x_154, 1); lean_inc(x_155); lean_dec(x_154); -x_156 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__99; +x_156 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__99; x_157 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_148, x_156, x_155); return x_157; } @@ -12424,205 +12421,205 @@ l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegi lean_mark_persistent(l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__74); l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__75 = _init_l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__75(); lean_mark_persistent(l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__75); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__1 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__1(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__1); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__2 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__2(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__2); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__3 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__3(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__3); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__4 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__4(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__4); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__5 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__5(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__5); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__6 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__6(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__6); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__7 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__7(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__7); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__8 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__8(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__8); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__9 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__9(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__9); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__10 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__10(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__10); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__11 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__11(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__11); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__12 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__12(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__12); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__13 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__13(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__13); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__14 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__14(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__14); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__15 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__15(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__15); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__16 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__16(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__16); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__17 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__17(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__17); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__18 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__18(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__18); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__19 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__19(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__19); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__20 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__20(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__20); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__21 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__21(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__21); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__22 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__22(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__22); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__23 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__23(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__23); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__24 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__24(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__24); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__25 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__25(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__25); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__26 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__26(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__26); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__27 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__27(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__27); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__28 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__28(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__28); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__29 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__29(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__29); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__30 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__30(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__30); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__31 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__31(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__31); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__32 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__32(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__32); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__33 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__33(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__33); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__34 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__34(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__34); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__35 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__35(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__35); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__36 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__36(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__36); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__37 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__37(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__37); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__38 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__38(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__38); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__39 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__39(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__39); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__40 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__40(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__40); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__41 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__41(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__41); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__42 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__42(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__42); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__43 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__43(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__43); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__44 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__44(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__44); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__45 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__45(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__45); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__46 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__46(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__46); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__47 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__47(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__47); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__48 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__48(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__48); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__49 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__49(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__49); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__50 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__50(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__50); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__51 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__51(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__51); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__52 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__52(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__52); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__53 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__53(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__53); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__54 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__54(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__54); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__55 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__55(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__55); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__56 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__56(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__56); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__57 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__57(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__57); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__58 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__58(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__58); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__59 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__59(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__59); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__60 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__60(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__60); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__61 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__61(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__61); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__62 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__62(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__62); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__63 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__63(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__63); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__64 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__64(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__64); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__65 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__65(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__65); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__66 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__66(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__66); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__67 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__67(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__67); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__68 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__68(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__68); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__69 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__69(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__69); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__70 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__70(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__70); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__71 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__71(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__71); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__72 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__72(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__72); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__73 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__73(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__73); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__74 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__74(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__74); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__75 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__75(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__75); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__76 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__76(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__76); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__77 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__77(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__77); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__78 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__78(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__78); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__79 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__79(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__79); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__80 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__80(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__80); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__81 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__81(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__81); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__82 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__82(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__82); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__83 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__83(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__83); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__84 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__84(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__84); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__85 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__85(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__85); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__86 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__86(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__86); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__87 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__87(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__87); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__88 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__88(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__88); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__89 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__89(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__89); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__90 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__90(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__90); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__91 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__91(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__91); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__92 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__92(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__92); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__93 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__93(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__93); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__94 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__94(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__94); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__95 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__95(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__95); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__96 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__96(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__96); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__97 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__97(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__97); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__98 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__98(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__98); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__99 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__99(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__99); -if (builtin) {res = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789_(lean_io_mk_world()); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__1 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__1(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__1); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__2 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__2(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__2); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__3 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__3(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__3); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__4 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__4(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__4); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__5 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__5(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__5); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__6 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__6(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__6); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__7 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__7(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__7); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__8 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__8(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__8); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__9 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__9(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__9); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__10 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__10(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__10); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__11 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__11(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__11); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__12 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__12(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__12); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__13 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__13(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__13); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__14 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__14(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__14); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__15 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__15(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__15); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__16 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__16(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__16); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__17 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__17(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__17); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__18 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__18(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__18); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__19 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__19(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__19); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__20 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__20(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__20); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__21 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__21(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__21); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__22 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__22(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__22); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__23 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__23(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__23); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__24 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__24(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__24); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__25 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__25(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__25); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__26 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__26(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__26); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__27 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__27(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__27); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__28 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__28(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__28); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__29 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__29(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__29); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__30 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__30(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__30); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__31 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__31(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__31); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__32 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__32(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__32); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__33 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__33(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__33); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__34 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__34(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__34); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__35 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__35(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__35); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__36 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__36(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__36); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__37 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__37(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__37); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__38 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__38(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__38); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__39 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__39(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__39); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__40 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__40(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__40); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__41 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__41(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__41); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__42 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__42(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__42); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__43 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__43(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__43); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__44 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__44(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__44); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__45 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__45(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__45); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__46 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__46(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__46); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__47 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__47(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__47); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__48 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__48(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__48); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__49 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__49(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__49); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__50 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__50(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__50); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__51 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__51(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__51); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__52 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__52(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__52); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__53 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__53(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__53); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__54 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__54(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__54); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__55 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__55(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__55); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__56 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__56(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__56); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__57 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__57(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__57); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__58 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__58(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__58); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__59 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__59(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__59); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__60 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__60(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__60); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__61 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__61(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__61); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__62 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__62(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__62); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__63 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__63(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__63); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__64 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__64(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__64); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__65 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__65(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__65); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__66 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__66(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__66); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__67 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__67(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__67); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__68 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__68(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__68); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__69 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__69(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__69); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__70 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__70(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__70); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__71 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__71(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__71); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__72 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__72(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__72); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__73 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__73(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__73); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__74 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__74(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__74); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__75 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__75(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__75); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__76 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__76(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__76); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__77 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__77(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__77); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__78 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__78(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__78); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__79 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__79(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__79); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__80 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__80(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__80); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__81 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__81(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__81); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__82 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__82(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__82); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__83 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__83(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__83); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__84 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__84(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__84); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__85 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__85(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__85); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__86 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__86(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__86); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__87 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__87(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__87); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__88 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__88(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__88); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__89 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__89(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__89); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__90 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__90(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__90); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__91 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__91(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__91); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__92 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__92(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__92); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__93 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__93(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__93); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__94 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__94(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__94); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__95 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__95(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__95); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__96 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__96(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__96); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__97 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__97(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__97); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__98 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__98(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__98); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__99 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__99(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__99); +if (builtin) {res = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }return lean_io_result_mk_ok(lean_box(0)); diff --git a/stage0/stdlib/Lean/Parser/Types.c b/stage0/stdlib/Lean/Parser/Types.c index 7c236366c2cd..2eaaab6177f1 100644 --- a/stage0/stdlib/Lean/Parser/Types.c +++ b/stage0/stdlib/Lean/Parser/Types.c @@ -27,6 +27,7 @@ static lean_object* l_Lean_Parser_instInhabitedError___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_ParserState_mkNode(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ParserState_setError(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Parser_withCacheFn___spec__4___at_Lean_Parser_withCacheFn___spec__5(lean_object*, lean_object*); +lean_object* l_Array_take___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_SyntaxStack_shrink___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Parser_withCacheFn___spec__6(lean_object*, lean_object*, lean_object*); uint32_t lean_string_utf8_get(lean_object*, lean_object*); @@ -108,6 +109,7 @@ static size_t l_Lean_PersistentHashMap_insertAux___at_Lean_Parser_SyntaxNodeKind LEAN_EXPORT lean_object* l_Lean_Parser_ParserState_popSyntax(lean_object*); static lean_object* l_Lean_Parser_SyntaxStack_back___closed__4; LEAN_EXPORT lean_object* l_panic___at_Lean_Parser_withCacheFn___spec__9(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Parser_ParserState_takeStack(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ParserState_stackSize___boxed(lean_object*); lean_object* lean_string_utf8_next(lean_object*, lean_object*); lean_object* l_String_decLt___boxed(lean_object*, lean_object*); @@ -213,7 +215,6 @@ LEAN_EXPORT uint8_t l___private_Lean_Parser_Types_0__Lean_Parser_beqCacheablePar LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Parser_withCacheFn___spec__1(lean_object*, lean_object*); LEAN_EXPORT uint32_t l_Lean_Parser_getNext(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ParserState_mkEOIError(lean_object*, lean_object*); -lean_object* l_Array_shrink___rarg(lean_object*, lean_object*); lean_object* l_Lean_PersistentHashMap_mkEmptyEntries(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Parser_withCacheFn___spec__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Parser_SyntaxNodeKindSet_insert___spec__3(size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -223,6 +224,7 @@ uint64_t lean_uint64_xor(uint64_t, uint64_t); extern lean_object* l_Id_instMonad; static lean_object* l_List_toString___at_Lean_Parser_FirstTokens_toStr___spec__1___closed__2; lean_object* lean_panic_fn(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Parser_SyntaxStack_take(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Parser_SyntaxStack_isEmpty(lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ParserState_next_x27(lean_object*, lean_object*, lean_object*, lean_object*); @@ -255,6 +257,7 @@ static lean_object* l_Lean_Parser_ParserFn_run___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_SyntaxStack_size___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Parser_Types_0__Lean_Parser_Error_expectedToString(lean_object*); size_t lean_usize_add(size_t, size_t); +LEAN_EXPORT lean_object* l_Lean_Parser_ParserState_takeStack___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Parser_SyntaxNodeKindSet_insert___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_instInhabitedParserInfo___lambda__1___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_withCacheFn___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -309,6 +312,7 @@ size_t lean_usize_land(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Parser_ParserState_mkErrorsAt(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ParserState_next_x27___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_toString___at_Lean_Parser_FirstTokens_toStr___spec__1___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Parser_SyntaxStack_take___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_FirstTokens_merge(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_mkAtom(lean_object* x_1, lean_object* x_2) { _start: @@ -1958,7 +1962,7 @@ x_3 = lean_box(x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Parser_SyntaxStack_shrink(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Parser_SyntaxStack_take(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; @@ -1969,7 +1973,7 @@ lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_4 = lean_ctor_get(x_1, 0); x_5 = lean_ctor_get(x_1, 1); x_6 = lean_nat_add(x_5, x_2); -x_7 = l_Array_shrink___rarg(x_4, x_6); +x_7 = l_Array_take___rarg(x_4, x_6); lean_dec(x_6); lean_ctor_set(x_1, 0, x_7); return x_1; @@ -1983,7 +1987,7 @@ lean_inc(x_9); lean_inc(x_8); lean_dec(x_1); x_10 = lean_nat_add(x_9, x_2); -x_11 = l_Array_shrink___rarg(x_8, x_10); +x_11 = l_Array_take___rarg(x_8, x_10); lean_dec(x_10); x_12 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_12, 0, x_11); @@ -1992,6 +1996,23 @@ return x_12; } } } +LEAN_EXPORT lean_object* l_Lean_Parser_SyntaxStack_take___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Lean_Parser_SyntaxStack_take(x_1, x_2); +lean_dec(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Parser_SyntaxStack_shrink(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Lean_Parser_SyntaxStack_take(x_1, x_2); +return x_3; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_SyntaxStack_shrink___boxed(lean_object* x_1, lean_object* x_2) { _start: { @@ -2110,7 +2131,7 @@ static lean_object* _init_l_Lean_Parser_SyntaxStack_back___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_Parser_SyntaxStack_back___closed__1; x_2 = l_Lean_Parser_SyntaxStack_back___closed__2; -x_3 = lean_unsigned_to_nat(176u); +x_3 = lean_unsigned_to_nat(178u); x_4 = lean_unsigned_to_nat(4u); x_5 = l_Lean_Parser_SyntaxStack_back___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -2173,7 +2194,7 @@ static lean_object* _init_l_Lean_Parser_SyntaxStack_get_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_Parser_SyntaxStack_back___closed__1; x_2 = l_Lean_Parser_SyntaxStack_get_x21___closed__1; -x_3 = lean_unsigned_to_nat(182u); +x_3 = lean_unsigned_to_nat(184u); x_4 = lean_unsigned_to_nat(4u); x_5 = l_Lean_Parser_SyntaxStack_get_x21___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -2394,7 +2415,7 @@ x_6 = lean_ctor_get(x_1, 4); lean_dec(x_6); x_7 = lean_ctor_get(x_1, 2); lean_dec(x_7); -x_8 = l_Lean_Parser_SyntaxStack_shrink(x_5, x_2); +x_8 = l_Lean_Parser_SyntaxStack_take(x_5, x_2); x_9 = lean_box(0); lean_ctor_set(x_1, 4, x_9); lean_ctor_set(x_1, 2, x_3); @@ -2413,7 +2434,7 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_dec(x_1); -x_14 = l_Lean_Parser_SyntaxStack_shrink(x_10, x_2); +x_14 = l_Lean_Parser_SyntaxStack_take(x_10, x_2); x_15 = lean_box(0); x_16 = lean_alloc_ctor(0, 6, 0); lean_ctor_set(x_16, 0, x_14); @@ -2593,7 +2614,7 @@ return x_12; } } } -LEAN_EXPORT lean_object* l_Lean_Parser_ParserState_shrinkStack(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Parser_ParserState_takeStack(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; @@ -2602,7 +2623,7 @@ if (x_3 == 0) { lean_object* x_4; lean_object* x_5; x_4 = lean_ctor_get(x_1, 0); -x_5 = l_Lean_Parser_SyntaxStack_shrink(x_4, x_2); +x_5 = l_Lean_Parser_SyntaxStack_take(x_4, x_2); lean_ctor_set(x_1, 0, x_5); return x_1; } @@ -2622,7 +2643,7 @@ lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_dec(x_1); -x_12 = l_Lean_Parser_SyntaxStack_shrink(x_6, x_2); +x_12 = l_Lean_Parser_SyntaxStack_take(x_6, x_2); x_13 = lean_alloc_ctor(0, 6, 0); lean_ctor_set(x_13, 0, x_12); lean_ctor_set(x_13, 1, x_7); @@ -2634,6 +2655,23 @@ return x_13; } } } +LEAN_EXPORT lean_object* l_Lean_Parser_ParserState_takeStack___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Lean_Parser_ParserState_takeStack(x_1, x_2); +lean_dec(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Parser_ParserState_shrinkStack(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Lean_Parser_ParserState_takeStack(x_1, x_2); +return x_3; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_ParserState_shrinkStack___boxed(lean_object* x_1, lean_object* x_2) { _start: { @@ -2771,7 +2809,7 @@ x_13 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_13, 0, x_12); lean_ctor_set(x_13, 1, x_2); lean_ctor_set(x_13, 2, x_11); -x_14 = l_Lean_Parser_SyntaxStack_shrink(x_5, x_3); +x_14 = l_Lean_Parser_SyntaxStack_take(x_5, x_3); x_15 = l_Lean_Parser_SyntaxStack_push(x_14, x_13); lean_ctor_set(x_1, 0, x_15); return x_1; @@ -2798,7 +2836,7 @@ x_21 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_21, 0, x_20); lean_ctor_set(x_21, 1, x_2); lean_ctor_set(x_21, 2, x_19); -x_22 = l_Lean_Parser_SyntaxStack_shrink(x_5, x_3); +x_22 = l_Lean_Parser_SyntaxStack_take(x_5, x_3); x_23 = l_Lean_Parser_SyntaxStack_push(x_22, x_21); lean_ctor_set(x_1, 0, x_23); return x_1; @@ -2838,7 +2876,7 @@ x_36 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_36, 0, x_35); lean_ctor_set(x_36, 1, x_2); lean_ctor_set(x_36, 2, x_34); -x_37 = l_Lean_Parser_SyntaxStack_shrink(x_24, x_3); +x_37 = l_Lean_Parser_SyntaxStack_take(x_24, x_3); x_38 = l_Lean_Parser_SyntaxStack_push(x_37, x_36); x_39 = lean_alloc_ctor(0, 6, 0); lean_ctor_set(x_39, 0, x_38); @@ -2877,7 +2915,7 @@ x_46 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_46, 0, x_45); lean_ctor_set(x_46, 1, x_2); lean_ctor_set(x_46, 2, x_44); -x_47 = l_Lean_Parser_SyntaxStack_shrink(x_24, x_3); +x_47 = l_Lean_Parser_SyntaxStack_take(x_24, x_3); x_48 = l_Lean_Parser_SyntaxStack_push(x_47, x_46); x_49 = lean_alloc_ctor(0, 6, 0); lean_ctor_set(x_49, 0, x_48); @@ -2919,7 +2957,7 @@ x_11 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_11, 0, x_10); lean_ctor_set(x_11, 1, x_2); lean_ctor_set(x_11, 2, x_9); -x_12 = l_Lean_Parser_SyntaxStack_shrink(x_5, x_7); +x_12 = l_Lean_Parser_SyntaxStack_take(x_5, x_7); lean_dec(x_7); x_13 = l_Lean_Parser_SyntaxStack_push(x_12, x_11); lean_ctor_set(x_1, 0, x_13); @@ -2951,7 +2989,7 @@ x_25 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_25, 0, x_24); lean_ctor_set(x_25, 1, x_2); lean_ctor_set(x_25, 2, x_23); -x_26 = l_Lean_Parser_SyntaxStack_shrink(x_14, x_21); +x_26 = l_Lean_Parser_SyntaxStack_take(x_14, x_21); lean_dec(x_21); x_27 = l_Lean_Parser_SyntaxStack_push(x_26, x_25); x_28 = lean_alloc_ctor(0, 6, 0); @@ -3275,7 +3313,7 @@ else { lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; x_8 = lean_ctor_get(x_4, 0); -x_9 = l_Lean_Parser_ParserState_shrinkStack(x_5, x_8); +x_9 = l_Lean_Parser_ParserState_takeStack(x_5, x_8); x_10 = lean_box(0); x_11 = l_Lean_Parser_ParserState_mkErrorsAt___lambda__1(x_2, x_9, x_10); return x_11; @@ -6081,7 +6119,7 @@ x_29 = l_Lean_Parser_instInhabitedInputContext___closed__2; x_30 = lean_string_append(x_28, x_29); x_31 = l_Lean_Parser_SyntaxStack_back___closed__1; x_32 = l_Lean_Parser_withCacheFn___lambda__2___closed__3; -x_33 = lean_unsigned_to_nat(429u); +x_33 = lean_unsigned_to_nat(433u); x_34 = lean_unsigned_to_nat(4u); x_35 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_31, x_32, x_33, x_34, x_30); lean_dec(x_30); diff --git a/stage0/stdlib/Lean/PrettyPrinter/Delaborator/Builtins.c b/stage0/stdlib/Lean/PrettyPrinter/Delaborator/Builtins.c index 96bfca56a8db..c316cc6bf791 100644 --- a/stage0/stdlib/Lean/PrettyPrinter/Delaborator/Builtins.c +++ b/stage0/stdlib/Lean/PrettyPrinter/Delaborator/Builtins.c @@ -30,6 +30,7 @@ static lean_object* l_Lean_PrettyPrinter_Delaborator_coeDelaborator___lambda__3_ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delaborator_delabConstWithSignature_delabParams___spec__2(lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_unresolveNameGlobal___at_Lean_PrettyPrinter_Delaborator_delabConst___spec__1___lambda__1___closed__1; static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabCond__1___closed__1; +static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__9___closed__2; lean_object* lean_string_utf8_extract(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_withMDataOptions___spec__8___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_withMDataOptions___spec__11(lean_object*); @@ -113,6 +114,7 @@ LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withBindingBod static lean_object* l_Lean_PrettyPrinter_Delaborator_delabDoElems___closed__5; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_PrettyPrinter_Delaborator_delabLam___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_pp_fullNames; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabConstWithSignature_delabParamsAux___lambda__15___closed__2; LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_delabProj___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabLam___lambda__3___closed__2; @@ -124,7 +126,9 @@ LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_instInhabitedParamKind static lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppMatch___lambda__6___closed__3; static lean_object* l_Lean_PrettyPrinter_Delaborator_unexpandStructureInstance___lambda__8___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delaborator_delabConstWithSignature_delabParamsAux___spec__13(lean_object*, lean_object*, size_t, size_t, lean_object*); +lean_object* l_Lean_Expr_name_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppImplicitCore_tryAppUnexpanders(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__5___closed__2; lean_object* lean_whnf(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_coeDelaborator___lambda__3___closed__1; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabDIte___lambda__1___closed__9; @@ -155,7 +159,6 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_declSigWi static lean_object* l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__8; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabConst___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabConstWithSignature_delabParamsAux___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabFVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_unresolveNameGlobal___at_Lean_PrettyPrinter_Delaborator_delabConst___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppImplicitCore___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -207,6 +210,7 @@ lean_object* l_Lean_Parser_leadingNode(lean_object*, lean_object*, lean_object*) LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withMDataExpr___at_Lean_PrettyPrinter_Delaborator_withMDataOptions___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___regBuiltin_Lean_PrettyPrinter_Delaborator_delabSort__1___closed__1; LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_delabMData___spec__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_PrettyPrinter_Delaborator_delabDo___closed__3; lean_object* l_Lean_Syntax_getId(lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabDivRatCore___closed__6; LEAN_EXPORT lean_object* l___private_Lean_PrettyPrinter_Delaborator_Builtins_0__Lean_PrettyPrinter_Delaborator_skippingBinders_loop_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*, lean_object*, lean_object*, lean_object*); @@ -235,17 +239,16 @@ LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_delabProj__ static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabMData__1___closed__3; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withBindingBody_x27___at_Lean_PrettyPrinter_Delaborator_delabDIte_delabBranch___spec__2___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withAppFn___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabDelayedAssignedMVar___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabApp___closed__1; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppExplicitCore___closed__4; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabChar___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabSigmaCore___lambda__1___closed__7; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabDoElems___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*); -uint8_t l_Array_contains___at_Lean_findField_x3f___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabLam___lambda__1___closed__2; static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabLetE__1___closed__5; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppImplicitCore_mkArg___closed__1; +static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__8___closed__2; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabDivRatCore___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_withMDatasOptions(lean_object*); lean_object* lean_mk_array(lean_object*, lean_object*); @@ -278,6 +281,7 @@ LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withBoundedApp LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__21(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabLetE___closed__1; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabLetFun(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__2; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabConst___closed__13; static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabLit__1___closed__3; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabConst___closed__9; @@ -424,7 +428,6 @@ static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabLam__1___ lean_object* l_Lean_getPPUniverses___boxed(lean_object*); static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabMData__1___closed__2; uint8_t l_Lean_Name_isPrefixOf(lean_object*, lean_object*); -static lean_object* l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__2; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabConstWithSignature_delabParamsAux___lambda__18(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_x27_loop___at_Lean_PrettyPrinter_Delaborator_unexpandStructureInstance___spec__1___closed__4; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_PrettyPrinter_Delaborator_delabAppImplicitCore_tryAppUnexpanders_go___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -512,6 +515,7 @@ static lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppMatch___lambda__6__ size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_useAppExplicit___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_isSubobjectField_x3f(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_PrettyPrinter_Delaborator_delabCond___closed__4; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppImplicitCore_mkArg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabDoElems___lambda__6___closed__3; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabLetE___closed__2; @@ -546,7 +550,6 @@ LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabDoElems___lambda_ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delaborator_delabConstWithSignature_delabParamsAux___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_getConstInfo___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__2___closed__4; static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabBVar__1___closed__5; -lean_object* l_Lean_Name_mkStr7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabFVar__1___closed__8; lean_object* l_Lean_Meta_withLocalDecl___at_Lean_PrettyPrinter_Delaborator_withBindingBodyUnusedName___spec__3___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabLam___lambda__3___closed__3; @@ -654,6 +657,7 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delabora extern lean_object* l_Lean_SubExpr_Pos_typeCoord; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabConstWithSignature_delabParamsAux___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_PrettyPrinter_Delaborator_delabLam___lambda__3___closed__8; +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_coeDelaborator___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabLetFun___lambda__2___closed__1; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppExplicitCore___lambda__3___closed__2; static lean_object* l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__5; @@ -665,7 +669,6 @@ LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabCond(lean_object* static lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppMatch___lambda__6___closed__6; LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_withMDataOptions___spec__3(lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_maybeAddBlockImplicit___closed__3; -static lean_object* l_Lean_PrettyPrinter_Delaborator_reifyName___closed__8; static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabHDiv__1___closed__4; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabDoElems___lambda__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabSort___closed__7; @@ -723,7 +726,7 @@ lean_object* l_Lean_getPPUnicodeFun___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabConstWithSignature_delabParamsAux___lambda__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabPProdMkCore___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_PrettyPrinter_Delaborator_delabConstWithSignature___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_coeDelaborator___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_coeDelaborator___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_appFieldNotationCandidate_x3f___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabDoElems___lambda__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabPSigma__1___closed__1; @@ -732,6 +735,7 @@ LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withAppArg___a lean_object* l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabMData(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_pp_universes; +static lean_object* l_Lean_PrettyPrinter_Delaborator_delabNeg___closed__3; 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_PrettyPrinter_Delaborator_delabDIte___closed__3; uint8_t l_List_isEmpty___rarg(lean_object*); @@ -756,7 +760,6 @@ uint8_t l_Lean_Expr_hasLooseBVars(lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabConstWithSignature_delabParamsAux___lambda__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_PrettyPrinter_Delaborator_Builtins_0__Lean_PrettyPrinter_Delaborator_evalSyntaxConstantUnsafe___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabForall___lambda__2___closed__3; -lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabOfNat__1(lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppExplicitCore___lambda__8___closed__2; lean_object* l_Lean_Syntax_node3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -766,6 +769,7 @@ LEAN_EXPORT lean_object* l___private_Lean_PrettyPrinter_Delaborator_Builtins_0__ static lean_object* l_Lean_PrettyPrinter_Delaborator_delabConst___closed__14; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabSigmaCore___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_append(lean_object*, lean_object*); +static lean_object* l_Lean_PrettyPrinter_Delaborator_delabOfNat___closed__7; LEAN_EXPORT lean_object* l___private_Lean_PrettyPrinter_Delaborator_Builtins_0__Lean_PrettyPrinter_Delaborator_withoutParentProjections___rarg(uint8_t, 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_x27___at___private_Lean_PrettyPrinter_Delaborator_Builtins_0__Lean_PrettyPrinter_Delaborator_skippingBinders_loop_visitLambda___spec__8(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_withMDataOptions___spec__8(lean_object*); @@ -776,6 +780,7 @@ LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabMVarAux___lambda_ static lean_object* l_Std_Range_forIn_loop___at_Lean_PrettyPrinter_Delaborator_getParamKinds___spec__1___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__22(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* l_Lean_PrettyPrinter_Delaborator_annotateTermInfo___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__1; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__3; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabDIte___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_descend___at___private_Lean_PrettyPrinter_Delaborator_Builtins_0__Lean_PrettyPrinter_Delaborator_skippingBinders_loop_visitLambda___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -813,7 +818,6 @@ static lean_object* l_Lean_PrettyPrinter_Delaborator_delabSort___closed__4; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_unexpandStructureInstance___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_declSigWithId_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_BinderInfo_isInstImplicit(uint8_t); -static lean_object* l_Lean_PrettyPrinter_Delaborator_reifyName___closed__7; LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabLetFun__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_unexpandStructureInstance___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabDIte___lambda__1___closed__2; @@ -844,6 +848,7 @@ static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabCond__1__ static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabFVar__1___closed__5; static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabPSigma__1___closed__3; static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__2; +static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__6___closed__2; static lean_object* l_Lean_PrettyPrinter_Delaborator_unexpandStructureInstance___lambda__8___closed__3; static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabPSigma__1___closed__2; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabForall___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -902,6 +907,7 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delabora uint8_t l_Lean_Syntax_matchesNull(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabLam__1(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delaborator_delabLam___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withMDataExpr___at_Lean_PrettyPrinter_Delaborator_withMDataOptions___spec__2___rarg___closed__3; LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_withMDataOptions___spec__10___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppMatch_withDummyBinders___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -918,7 +924,6 @@ static lean_object* l_Lean_PrettyPrinter_Delaborator_delabLam___lambda__1___clos extern lean_object* l_Lean_diagnostics; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabDoElems(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_isIdent(lean_object*); -static lean_object* l_Lean_PrettyPrinter_Delaborator_reifyName___closed__12; lean_object* l_Lean_SubExpr_Pos_pushNaryArg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_unexpandStructureInstance___lambda__3___closed__6; static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__1; @@ -981,7 +986,6 @@ static lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppImplicitCore_mkName LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_descend___at___private_Lean_PrettyPrinter_Delaborator_Builtins_0__Lean_PrettyPrinter_Delaborator_skippingBinders_loop_visitLambda___spec__3(lean_object*); static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabDo__1___closed__2; lean_object* l_Lean_MessageData_ofExpr(lean_object*); -static lean_object* l_Lean_PrettyPrinter_Delaborator_reifyName___closed__3; static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__3; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabMVarAux___closed__1; lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withType___at_Lean_PrettyPrinter_Delaborator_delab___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1018,12 +1022,10 @@ static lean_object* l___private_Lean_PrettyPrinter_Delaborator_Builtins_0__Lean_ lean_object* l_Lean_LocalDecl_userName(lean_object*); lean_object* l_Lean_getPPMVarsWithType___boxed(lean_object*); lean_object* l_Array_extract___rarg(lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Name_mkStr6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_node4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabMProdMk__1(lean_object*); uint8_t l_Lean_Expr_isAutoParam(lean_object*); lean_object* l_Lean_getPPMVarsAnonymous___boxed(lean_object*); -static lean_object* l_Lean_PrettyPrinter_Delaborator_reifyName___closed__2; static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_declSigWithId_formatter__1___closed__2; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppImplicitCore___lambda__12___closed__1; static lean_object* l_Lean_PrettyPrinter_Delaborator_coeDelaborator___lambda__2___closed__1; @@ -1040,7 +1042,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeReducing___at___private_Lean LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__4(lean_object*); static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabProj__1___closed__4; static lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withBindingBody___at___private_Lean_PrettyPrinter_Delaborator_Builtins_0__Lean_PrettyPrinter_Delaborator_skippingBinders_loop_visitLambda___spec__1___rarg___closed__1; -static lean_object* l_Lean_PrettyPrinter_Delaborator_reifyName___closed__5; static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__2___closed__1; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabConstWithSignature_delabParams___closed__6; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabHDiv(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1097,6 +1098,7 @@ lean_object* l_Lean_Name_appendCore(lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppImplicitCore_mkNamedArg___closed__1; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabSigmaCore___lambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppExplicitCore___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__2___closed__2; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabLam___lambda__1___closed__7; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_unexpandStructureInstance___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabPProdMk__1___closed__3; @@ -1108,6 +1110,7 @@ LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withBindingBod LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_PrettyPrinter_Delaborator_needsExplicit___spec__2(lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabSigmaCore___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabDo___closed__1; +static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__5; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withNaryArg___at_Lean_PrettyPrinter_Delaborator_delabLetFun___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_Delaborator_returnsPi___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_unexpandStructureInstance___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1119,6 +1122,7 @@ static lean_object* l_Lean_PrettyPrinter_Delaborator_delabConstWithSignature_del LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withBindingBody_x27___at___private_Lean_PrettyPrinter_Delaborator_Builtins_0__Lean_PrettyPrinter_Delaborator_shouldGroupWithNext___spec__2___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabSort___closed__13; LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_withMDataOptions___spec__12___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__7___closed__2; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_needsExplicit___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__9; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_declSigWithId_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1132,7 +1136,6 @@ uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_x27___s static lean_object* l_Lean_PrettyPrinter_Delaborator_delabCond___closed__1; lean_object* l_Lean_getPPPiBinderTypes___boxed(lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabLetFun___lambda__2___closed__4; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_coeDelaborator___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__3; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabSort___closed__12; @@ -1157,7 +1160,6 @@ LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabDoElems_prependAn lean_object* l_Lean_PrettyPrinter_Delaborator_failure___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabDIte_delabBranch___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_PrettyPrinter_Delaborator_Builtins_0__Lean_PrettyPrinter_Delaborator_withoutParentProjections___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_PrettyPrinter_Delaborator_unexpandStructureInstance___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_delabProj___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_withCache(lean_object*, lean_object*); @@ -1197,15 +1199,15 @@ LEAN_EXPORT lean_object* l___private_Lean_PrettyPrinter_Delaborator_Builtins_0__ static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabAppMatch__1___closed__3; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_PrettyPrinter_Delaborator_needsExplicit___spec__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabForall___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__5; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delaborator_delabConstWithSignature_delabParamsAux___spec__4(lean_object*, lean_object*, size_t, size_t, lean_object*); -static lean_object* l_Lean_PrettyPrinter_Delaborator_reifyName___closed__11; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withBindingBody_x27___at___private_Lean_PrettyPrinter_Delaborator_Builtins_0__Lean_PrettyPrinter_Delaborator_skippingBinders_loop_visitLambda___spec__2(lean_object*, lean_object*); -static lean_object* l_Lean_PrettyPrinter_Delaborator_reifyName___closed__4; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppImplicitCore_mkArg___closed__2; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppExplicitCore___closed__1; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabProj___closed__1; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabConstWithSignature_delabParamsAux___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_node1(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_PrettyPrinter_Delaborator_delabOfScientific___closed__4; static lean_object* l_Lean_PrettyPrinter_Delaborator_unexpandStructureInstance___lambda__3___closed__5; lean_object* l_Lean_Parser_Command_declSig_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabPSigma__1___closed__4; @@ -1233,8 +1235,10 @@ LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppExplicitCore__ static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabFVar__1___closed__4; lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabMVarAux___lambda__1___closed__7; +uint8_t l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(lean_object*, lean_object*); lean_object* l_Lean_Level_dec(lean_object*); uint8_t l_Lean_Syntax_hasIdent(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_coeDelaborator___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabLetFun___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_type(lean_object*); static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabFVar__1___closed__3; @@ -1318,7 +1322,6 @@ extern lean_object* l_Lean_Parser_maxPrec; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delaborator_delabConstWithSignature_delabParamsAux___spec__5(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withBindingBody_x27___at_Lean_PrettyPrinter_Delaborator_delabAppMatch_usingNames___spec__2___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabDivRatCore___closed__1; -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_reifyName(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_PrettyPrinter_Delaborator_Builtins_0__Lean_PrettyPrinter_Delaborator_stripParentProjections___closed__1; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabDoElems___lambda__1___closed__2; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabLetE___closed__4; @@ -1327,7 +1330,6 @@ LEAN_EXPORT lean_object* l_Lean_unresolveNameGlobal_unresolveNameCore___at_Lean_ lean_object* l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); lean_object* l_Array_ofSubarray___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabConstWithSignature_delabParamsAux___lambda__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_PrettyPrinter_Delaborator_reifyName___closed__6; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabSigmaCore___lambda__1___closed__1; uint8_t l_Lean_LocalDecl_binderInfo(lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabOfScientific___closed__3; @@ -1337,6 +1339,7 @@ static lean_object* l_Lean_PrettyPrinter_Delaborator_useAppExplicit___lambda__2_ LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withBindingBody_x27___at___private_Lean_PrettyPrinter_Delaborator_Builtins_0__Lean_PrettyPrinter_Delaborator_skippingBinders_loop_visitLambda___spec__8___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_delabMData___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabNeg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__4___closed__2; lean_object* lean_erase_macro_scopes(lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabOfScientific___lambda__1___closed__3; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -1345,6 +1348,7 @@ lean_object* l_Array_back___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_delabMData___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppImplicitCore___closed__2; static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabChar__1___closed__4; +static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__6; LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_delabMData___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delaborator_delabConstWithSignature_delabParams___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withBindingBody_x27___at___private_Lean_PrettyPrinter_Delaborator_Builtins_0__Lean_PrettyPrinter_Delaborator_skippingBinders_loop_visitLambda___spec__5___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1358,6 +1362,7 @@ size_t lean_usize_sub(size_t, size_t); static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabLam__1___closed__1; lean_object* lean_array_mk(lean_object*); static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabForall__1___closed__5; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppImplicitCore___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppMatch___lambda__3___closed__4; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabNegIntCore___closed__7; @@ -1379,7 +1384,6 @@ size_t lean_usize_add(size_t, size_t); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppMatch___closed__4; static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_declSigWithId_parenthesizer__1___closed__2; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppCore___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__1; static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabPProdMk__1___closed__4; LEAN_EXPORT uint8_t l_Lean_PrettyPrinter_Delaborator_delabAppImplicitCore___lambda__3(lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabApp___lambda__2(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1419,7 +1423,6 @@ extern lean_object* l_Lean_instInhabitedSyntax; lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_useAppExplicit___closed__1; LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_withMDataOptions___spec__10(lean_object*); -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_reifyName___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_PrettyPrinter_Delaborator_Builtins_0__Lean_PrettyPrinter_Delaborator_delabBinders___closed__1; lean_object* l_Lean_SubExpr_Pos_pushNaryFn(lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_Delaborator_addFieldInfo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1435,11 +1438,12 @@ lean_object* l_Lean_Expr_bindingBody_x21(lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabLam___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_PrettyPrinter_Delaborator_delabLit__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeReducing___at___private_Lean_PrettyPrinter_Delaborator_Builtins_0__Lean_PrettyPrinter_Delaborator_skippingBinders_loop___spec__1___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_PrettyPrinter_Delaborator_delabHDiv___closed__3; lean_object* l_Lean_getPPExplicit___boxed(lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_getParamKinds___closed__1; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabDo___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabForall__1___closed__4; -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_coeDelaborator___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_coeDelaborator___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppImplicitCore___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabDIte__1___closed__2; @@ -1467,7 +1471,6 @@ LEAN_EXPORT lean_object* l_Lean_resolveGlobalName___at_Lean_PrettyPrinter_Delabo static lean_object* l_Lean_PrettyPrinter_Delaborator_delabSort___closed__1; static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_declSigWithId_parenthesizer__1___closed__4; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabForall___lambda__2___closed__1; -static lean_object* l_Lean_PrettyPrinter_Delaborator_reifyName___closed__9; lean_object* l_Lean_PrettyPrinter_Delaborator_withBindingBodyUnusedName___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppMatch___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1501,7 +1504,6 @@ uint8_t l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_404_( LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_PrettyPrinter_Delaborator_getParamKinds___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNeg__1___closed__3; LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabDIte__1(lean_object*); -static lean_object* l_Lean_PrettyPrinter_Delaborator_reifyName___closed__10; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delaborator_delabConst___spec__6(uint8_t, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delaborator_delabConst___spec__7(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_declSigWithId_formatter__1(lean_object*); @@ -1594,10 +1596,12 @@ static lean_object* l___private_Lean_PrettyPrinter_Delaborator_Builtins_0__Lean_ LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_withMDataOptions___spec__7___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delaborator_delabConstWithSignature_delabParams___spec__1(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppMatch___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__3___closed__2; lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallTelescopeReducingImp___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__5___closed__1; static lean_object* l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__6; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabDIte___lambda__1___closed__1; +static lean_object* l_Lean_PrettyPrinter_Delaborator_delabDIte___closed__4; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabDoElems___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_List_forIn_loop___at_Lean_PrettyPrinter_Delaborator_delabConst___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_unexpandStructureInstance___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*); @@ -1619,7 +1623,6 @@ static lean_object* l_Lean_PrettyPrinter_Delaborator_appFieldNotationCandidate_x static lean_object* l_Lean_PrettyPrinter_Delaborator_delabConst___closed__12; lean_object* l_Lean_Syntax_mkNumLit(lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabLam___lambda__1___closed__8; -lean_object* l_Lean_Name_mkStr8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_PrettyPrinter_Delaborator_delabConst___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withBindingBody___at___private_Lean_PrettyPrinter_Delaborator_Builtins_0__Lean_PrettyPrinter_Delaborator_shouldGroupWithNext___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -22912,7 +22915,7 @@ if (x_20 == 0) { uint8_t x_21; lean_dec(x_18); -x_21 = l_Array_contains___at_Lean_findField_x3f___spec__1(x_5, x_17); +x_21 = l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(x_5, x_17); if (x_21 == 0) { lean_object* x_22; lean_object* x_23; @@ -24671,7 +24674,7 @@ return x_24; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; @@ -24728,7 +24731,7 @@ return x_20; } } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__1() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__1() { _start: { lean_object* x_1; lean_object* x_2; @@ -24738,15 +24741,15 @@ lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__2() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__2() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___lambda__1), 8, 0); +x_1 = lean_alloc_closure((void*)(l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___lambda__1), 8, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { lean_object* x_16; uint8_t x_17; @@ -24776,8 +24779,8 @@ x_24 = lean_ctor_get(x_1, 6); x_25 = lean_array_get_size(x_24); x_26 = lean_nat_dec_lt(x_6, x_25); lean_dec(x_25); -x_27 = l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__1; -x_28 = l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__2; +x_27 = l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__1; +x_28 = l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__2; x_29 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Delaborator_SubExpr_withAppFnArgs___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__14), 9, 2); lean_closure_set(x_29, 0, x_27); lean_closure_set(x_29, 1, x_28); @@ -26640,7 +26643,7 @@ lean_dec(x_16); x_18 = lean_array_get_size(x_17); x_19 = lean_mk_empty_array_with_capacity(x_18); x_20 = lean_unsigned_to_nat(0u); -x_21 = l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18(x_1, x_14, x_17, x_17, x_18, x_20, lean_box(0), x_19, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_21 = l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18(x_1, x_14, x_17, x_17, x_18, x_20, lean_box(0), x_19, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_17); lean_dec(x_14); return x_21; @@ -28023,11 +28026,11 @@ lean_dec(x_4); return x_14; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { lean_object* x_16; -x_16 = l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +x_16 = l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); @@ -37661,13 +37664,25 @@ x_1 = lean_alloc_closure((void*)(l_Lean_getPPCoercions___boxed), 1, 0); return x_1; } } +static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_delabOfNat___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_PrettyPrinter_Delaborator_delabOfNat___closed__6; +x_2 = l_Lean_PrettyPrinter_Delaborator_delabOfNat___closed__5; +x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Delaborator_whenPPOption), 9, 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_Delaborator_delabOfNat(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; lean_object* x_9; lean_object* x_10; -x_8 = l_Lean_PrettyPrinter_Delaborator_delabOfNat___closed__6; -x_9 = l_Lean_PrettyPrinter_Delaborator_delabOfNat___closed__5; -x_10 = l_Lean_PrettyPrinter_Delaborator_whenPPOption(x_8, x_9, x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Lean_PrettyPrinter_Delaborator_useAppExplicit___closed__1; +x_9 = l_Lean_PrettyPrinter_Delaborator_delabOfNat___closed__7; +x_10 = l_Lean_PrettyPrinter_Delaborator_whenNotPPOption(x_8, x_9, x_1, x_2, x_3, x_4, x_5, x_6, x_7); return x_10; } } @@ -37742,13 +37757,25 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } +static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_delabNeg___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_PrettyPrinter_Delaborator_delabOfNat___closed__6; +x_2 = l_Lean_PrettyPrinter_Delaborator_delabNeg___closed__2; +x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Delaborator_whenPPOption), 9, 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_Delaborator_delabNeg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; lean_object* x_9; lean_object* x_10; -x_8 = l_Lean_PrettyPrinter_Delaborator_delabOfNat___closed__6; -x_9 = l_Lean_PrettyPrinter_Delaborator_delabNeg___closed__2; -x_10 = l_Lean_PrettyPrinter_Delaborator_whenPPOption(x_8, x_9, x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Lean_PrettyPrinter_Delaborator_useAppExplicit___closed__1; +x_9 = l_Lean_PrettyPrinter_Delaborator_delabNeg___closed__3; +x_10 = l_Lean_PrettyPrinter_Delaborator_whenNotPPOption(x_8, x_9, x_1, x_2, x_3, x_4, x_5, x_6, x_7); return x_10; } } @@ -37823,13 +37850,25 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } +static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_delabHDiv___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_PrettyPrinter_Delaborator_delabOfNat___closed__6; +x_2 = l_Lean_PrettyPrinter_Delaborator_delabHDiv___closed__2; +x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Delaborator_whenPPOption), 9, 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_Delaborator_delabHDiv(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; lean_object* x_9; lean_object* x_10; -x_8 = l_Lean_PrettyPrinter_Delaborator_delabOfNat___closed__6; -x_9 = l_Lean_PrettyPrinter_Delaborator_delabHDiv___closed__2; -x_10 = l_Lean_PrettyPrinter_Delaborator_whenPPOption(x_8, x_9, x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Lean_PrettyPrinter_Delaborator_useAppExplicit___closed__1; +x_9 = l_Lean_PrettyPrinter_Delaborator_delabHDiv___closed__3; +x_10 = l_Lean_PrettyPrinter_Delaborator_whenNotPPOption(x_8, x_9, x_1, x_2, x_3, x_4, x_5, x_6, x_7); return x_10; } } @@ -38413,13 +38452,25 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } +static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_delabOfScientific___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_PrettyPrinter_Delaborator_delabOfNat___closed__6; +x_2 = l_Lean_PrettyPrinter_Delaborator_delabOfScientific___closed__3; +x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Delaborator_whenPPOption), 9, 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_Delaborator_delabOfScientific(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; lean_object* x_9; lean_object* x_10; -x_8 = l_Lean_PrettyPrinter_Delaborator_delabOfNat___closed__6; -x_9 = l_Lean_PrettyPrinter_Delaborator_delabOfScientific___closed__3; -x_10 = l_Lean_PrettyPrinter_Delaborator_whenPPOption(x_8, x_9, x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Lean_PrettyPrinter_Delaborator_useAppExplicit___closed__1; +x_9 = l_Lean_PrettyPrinter_Delaborator_delabOfScientific___closed__4; +x_10 = l_Lean_PrettyPrinter_Delaborator_whenNotPPOption(x_8, x_9, x_1, x_2, x_3, x_4, x_5, x_6, x_7); return x_10; } } @@ -39270,7 +39321,98 @@ x_1 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Delaborator_coeDelaborator return x_1; } } -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_coeDelaborator___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_Lean_PrettyPrinter_Delaborator_coeDelaborator___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +uint8_t x_11; +x_11 = lean_ctor_get_uint8(x_1, sizeof(void*)*2); +switch (x_11) { +case 0: +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_12 = lean_ctor_get(x_1, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_1, 1); +lean_inc(x_13); +lean_dec(x_1); +x_14 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__1; +x_15 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Delaborator_SubExpr_withNaryArg___at_Lean_PrettyPrinter_Delaborator_delabLetFun___spec__5___boxed), 9, 2); +lean_closure_set(x_15, 0, x_13); +lean_closure_set(x_15, 1, x_14); +x_16 = l_Lean_PrettyPrinter_Delaborator_coeDelaborator___lambda__4___closed__1; +x_17 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_PrettyPrinter_Delaborator_delabMVarAux___spec__1___rarg), 9, 2); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_16); +x_18 = l_Lean_PrettyPrinter_Delaborator_withOverApp(x_12, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_12); +return x_18; +} +case 1: +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; +x_19 = lean_ctor_get(x_1, 0); +lean_inc(x_19); +x_20 = lean_unsigned_to_nat(0u); +x_21 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_20); +x_22 = lean_nat_dec_eq(x_21, x_19); +lean_dec(x_21); +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_inc(x_23); +lean_dec(x_1); +x_24 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__1; +x_25 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Delaborator_SubExpr_withNaryArg___at_Lean_PrettyPrinter_Delaborator_delabLetFun___spec__5___boxed), 9, 2); +lean_closure_set(x_25, 0, x_23); +lean_closure_set(x_25, 1, x_24); +x_26 = l_Lean_PrettyPrinter_Delaborator_withOverApp(x_19, x_25, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_19); +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_1, 1); +lean_inc(x_27); +lean_dec(x_1); +x_28 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__1; +x_29 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Delaborator_SubExpr_withNaryArg___at_Lean_PrettyPrinter_Delaborator_delabLetFun___spec__5___boxed), 9, 2); +lean_closure_set(x_29, 0, x_27); +lean_closure_set(x_29, 1, x_28); +x_30 = l_Lean_PrettyPrinter_Delaborator_coeDelaborator___lambda__4___closed__2; +x_31 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_PrettyPrinter_Delaborator_delabMVarAux___spec__1___rarg), 9, 2); +lean_closure_set(x_31, 0, x_29); +lean_closure_set(x_31, 1, x_30); +x_32 = l_Lean_PrettyPrinter_Delaborator_withOverApp(x_19, x_31, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_19); +return x_32; +} +} +default: +{ +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_33 = lean_ctor_get(x_1, 0); +lean_inc(x_33); +x_34 = lean_ctor_get(x_1, 1); +lean_inc(x_34); +lean_dec(x_1); +x_35 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__1; +x_36 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Delaborator_SubExpr_withNaryArg___at_Lean_PrettyPrinter_Delaborator_delabLetFun___spec__5___boxed), 9, 2); +lean_closure_set(x_36, 0, x_34); +lean_closure_set(x_36, 1, x_35); +x_37 = l_Lean_PrettyPrinter_Delaborator_coeDelaborator___lambda__4___closed__3; +x_38 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_PrettyPrinter_Delaborator_delabMVarAux___spec__1___rarg), 9, 2); +lean_closure_set(x_38, 0, x_36); +lean_closure_set(x_38, 1, x_37); +x_39 = l_Lean_PrettyPrinter_Delaborator_withOverApp(x_33, x_38, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_33); +return x_39; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_coeDelaborator___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; @@ -39302,109 +39444,122 @@ return x_14; } else { -lean_object* x_15; uint8_t x_16; -x_15 = lean_ctor_get(x_12, 0); +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_15 = lean_ctor_get(x_11, 1); lean_inc(x_15); +lean_dec(x_11); +x_16 = lean_ctor_get(x_12, 0); +lean_inc(x_16); lean_dec(x_12); -x_16 = lean_ctor_get_uint8(x_15, sizeof(void*)*2); -switch (x_16) { -case 0: +x_17 = l_Lean_PrettyPrinter_Delaborator_useAppExplicit___closed__1; +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +x_18 = l_Lean_PrettyPrinter_Delaborator_getPPOption___rarg(x_17, x_2, x_3, x_4, x_5, x_6, x_7, x_15); +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; -x_17 = lean_ctor_get(x_11, 1); -lean_inc(x_17); -lean_dec(x_11); -x_18 = lean_ctor_get(x_15, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_15, 1); +lean_object* x_19; uint8_t x_20; +x_19 = lean_ctor_get(x_18, 0); lean_inc(x_19); -lean_dec(x_15); -x_20 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__1; -x_21 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Delaborator_SubExpr_withNaryArg___at_Lean_PrettyPrinter_Delaborator_delabLetFun___spec__5___boxed), 9, 2); -lean_closure_set(x_21, 0, x_19); -lean_closure_set(x_21, 1, x_20); -x_22 = l_Lean_PrettyPrinter_Delaborator_coeDelaborator___lambda__4___closed__1; -x_23 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_PrettyPrinter_Delaborator_delabMVarAux___spec__1___rarg), 9, 2); -lean_closure_set(x_23, 0, x_21); -lean_closure_set(x_23, 1, x_22); -x_24 = l_Lean_PrettyPrinter_Delaborator_withOverApp(x_18, x_23, x_2, x_3, x_4, x_5, x_6, x_7, x_17); +x_20 = lean_unbox(x_19); +lean_dec(x_19); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_18, 1); +lean_inc(x_21); lean_dec(x_18); -return x_24; +x_22 = lean_box(0); +x_23 = l_Lean_PrettyPrinter_Delaborator_coeDelaborator___lambda__4(x_16, x_1, x_22, x_2, x_3, x_4, x_5, x_6, x_7, x_21); +return x_23; } -case 1: +else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; -x_25 = lean_ctor_get(x_11, 1); +lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; +x_24 = lean_ctor_get(x_18, 1); +lean_inc(x_24); +lean_dec(x_18); +x_25 = lean_ctor_get(x_16, 1); lean_inc(x_25); -lean_dec(x_11); -x_26 = lean_ctor_get(x_15, 0); -lean_inc(x_26); -x_27 = lean_unsigned_to_nat(0u); -x_28 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_27); -x_29 = lean_nat_dec_eq(x_28, x_26); -lean_dec(x_28); +x_26 = lean_unsigned_to_nat(0u); +x_27 = lean_nat_dec_eq(x_25, x_26); +lean_dec(x_25); +if (x_27 == 0) +{ +lean_object* x_28; uint8_t x_29; +lean_dec(x_16); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_28 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_24); +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; -x_30 = lean_ctor_get(x_15, 1); +return x_28; +} +else +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_28, 0); +x_31 = lean_ctor_get(x_28, 1); +lean_inc(x_31); lean_inc(x_30); -lean_dec(x_15); -x_31 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__1; -x_32 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Delaborator_SubExpr_withNaryArg___at_Lean_PrettyPrinter_Delaborator_delabLetFun___spec__5___boxed), 9, 2); -lean_closure_set(x_32, 0, x_30); -lean_closure_set(x_32, 1, x_31); -x_33 = l_Lean_PrettyPrinter_Delaborator_withOverApp(x_26, x_32, x_2, x_3, x_4, x_5, x_6, x_7, x_25); -lean_dec(x_26); -return x_33; +lean_dec(x_28); +x_32 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_31); +return x_32; +} } else { -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_34 = lean_ctor_get(x_15, 1); -lean_inc(x_34); -lean_dec(x_15); -x_35 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__1; -x_36 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Delaborator_SubExpr_withNaryArg___at_Lean_PrettyPrinter_Delaborator_delabLetFun___spec__5___boxed), 9, 2); -lean_closure_set(x_36, 0, x_34); -lean_closure_set(x_36, 1, x_35); -x_37 = l_Lean_PrettyPrinter_Delaborator_coeDelaborator___lambda__4___closed__2; -x_38 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_PrettyPrinter_Delaborator_delabMVarAux___spec__1___rarg), 9, 2); -lean_closure_set(x_38, 0, x_36); -lean_closure_set(x_38, 1, x_37); -x_39 = l_Lean_PrettyPrinter_Delaborator_withOverApp(x_26, x_38, x_2, x_3, x_4, x_5, x_6, x_7, x_25); -lean_dec(x_26); -return x_39; +lean_object* x_33; lean_object* x_34; +x_33 = lean_box(0); +x_34 = l_Lean_PrettyPrinter_Delaborator_coeDelaborator___lambda__4(x_16, x_1, x_33, x_2, x_3, x_4, x_5, x_6, x_7, x_24); +return x_34; } } -default: +} +else { -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_40 = lean_ctor_get(x_11, 1); -lean_inc(x_40); -lean_dec(x_11); -x_41 = lean_ctor_get(x_15, 0); -lean_inc(x_41); -x_42 = lean_ctor_get(x_15, 1); -lean_inc(x_42); -lean_dec(x_15); -x_43 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__1; -x_44 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Delaborator_SubExpr_withNaryArg___at_Lean_PrettyPrinter_Delaborator_delabLetFun___spec__5___boxed), 9, 2); -lean_closure_set(x_44, 0, x_42); -lean_closure_set(x_44, 1, x_43); -x_45 = l_Lean_PrettyPrinter_Delaborator_coeDelaborator___lambda__4___closed__3; -x_46 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_PrettyPrinter_Delaborator_delabMVarAux___spec__1___rarg), 9, 2); -lean_closure_set(x_46, 0, x_44); -lean_closure_set(x_46, 1, x_45); -x_47 = l_Lean_PrettyPrinter_Delaborator_withOverApp(x_41, x_46, x_2, x_3, x_4, x_5, x_6, x_7, x_40); -lean_dec(x_41); -return x_47; +uint8_t x_35; +lean_dec(x_16); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_35 = !lean_is_exclusive(x_18); +if (x_35 == 0) +{ +return x_18; +} +else +{ +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_18, 0); +x_37 = lean_ctor_get(x_18, 1); +lean_inc(x_37); +lean_inc(x_36); +lean_dec(x_18); +x_38 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_38, 0, x_36); +lean_ctor_set(x_38, 1, x_37); +return x_38; } } } } else { -lean_object* x_48; +lean_object* x_39; lean_dec(x_9); lean_dec(x_7); lean_dec(x_6); @@ -39412,8 +39567,8 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_48 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_48; +x_39 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); +return x_39; } } } @@ -39421,7 +39576,7 @@ static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_coeDelaborator___clos _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Delaborator_coeDelaborator___lambda__4___boxed), 8, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Delaborator_coeDelaborator___lambda__5___boxed), 8, 0); return x_1; } } @@ -39489,11 +39644,21 @@ lean_dec(x_2); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_coeDelaborator___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_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_coeDelaborator___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_PrettyPrinter_Delaborator_coeDelaborator___lambda__4(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; +} +} +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_coeDelaborator___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: { lean_object* x_9; -x_9 = l_Lean_PrettyPrinter_Delaborator_coeDelaborator___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_PrettyPrinter_Delaborator_coeDelaborator___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_1); return x_9; } @@ -40525,13 +40690,25 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } +static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_delabDIte___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_PrettyPrinter_Delaborator_delabAppImplicitCore___lambda__11___closed__2; +x_2 = l_Lean_PrettyPrinter_Delaborator_delabDIte___closed__3; +x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Delaborator_whenPPOption), 9, 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_Delaborator_delabDIte(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; lean_object* x_9; lean_object* x_10; -x_8 = l_Lean_PrettyPrinter_Delaborator_delabAppImplicitCore___lambda__11___closed__2; -x_9 = l_Lean_PrettyPrinter_Delaborator_delabDIte___closed__3; -x_10 = l_Lean_PrettyPrinter_Delaborator_whenPPOption(x_8, x_9, x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Lean_PrettyPrinter_Delaborator_useAppExplicit___closed__1; +x_9 = l_Lean_PrettyPrinter_Delaborator_delabDIte___closed__4; +x_10 = l_Lean_PrettyPrinter_Delaborator_whenNotPPOption(x_8, x_9, x_1, x_2, x_3, x_4, x_5, x_6, x_7); return x_10; } } @@ -40899,13 +41076,25 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } +static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_delabCond___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_PrettyPrinter_Delaborator_delabAppImplicitCore___lambda__11___closed__2; +x_2 = l_Lean_PrettyPrinter_Delaborator_delabCond___closed__3; +x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Delaborator_whenPPOption), 9, 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_Delaborator_delabCond(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; lean_object* x_9; lean_object* x_10; -x_8 = l_Lean_PrettyPrinter_Delaborator_delabAppImplicitCore___lambda__11___closed__2; -x_9 = l_Lean_PrettyPrinter_Delaborator_delabCond___closed__3; -x_10 = l_Lean_PrettyPrinter_Delaborator_whenPPOption(x_8, x_9, x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Lean_PrettyPrinter_Delaborator_useAppExplicit___closed__1; +x_9 = l_Lean_PrettyPrinter_Delaborator_delabCond___closed__4; +x_10 = l_Lean_PrettyPrinter_Delaborator_whenNotPPOption(x_8, x_9, x_1, x_2, x_3, x_4, x_5, x_6, x_7); return x_10; } } @@ -42083,7 +42272,7 @@ return x_25; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabSigmaCore(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) { _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_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; x_9 = lean_box(x_1); x_10 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Delaborator_delabSigmaCore___lambda__3___boxed), 9, 1); lean_closure_set(x_10, 0, x_9); @@ -42092,8 +42281,12 @@ x_12 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_PrettyPrinter_Delabor lean_closure_set(x_12, 0, x_11); lean_closure_set(x_12, 1, x_10); x_13 = l_Lean_PrettyPrinter_Delaborator_delabAppImplicitCore___lambda__11___closed__2; -x_14 = l_Lean_PrettyPrinter_Delaborator_whenPPOption(x_13, x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -return x_14; +x_14 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Delaborator_whenPPOption), 9, 2); +lean_closure_set(x_14, 0, x_13); +lean_closure_set(x_14, 1, x_12); +x_15 = l_Lean_PrettyPrinter_Delaborator_useAppExplicit___closed__1; +x_16 = l_Lean_PrettyPrinter_Delaborator_whenNotPPOption(x_15, x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +return x_16; } } LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabSigmaCore___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { @@ -43596,7 +43789,7 @@ static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_delabDoElems___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_PrettyPrinter_Delaborator_delabFVar___closed__1; x_2 = l_Lean_PrettyPrinter_Delaborator_delabDoElems___closed__4; -x_3 = lean_unsigned_to_nat(1187u); +x_3 = lean_unsigned_to_nat(1190u); x_4 = lean_unsigned_to_nat(40u); x_5 = l_Lean_PrettyPrinter_Delaborator_delabFVar___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -44990,13 +45183,25 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } +static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_delabDo___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_PrettyPrinter_Delaborator_delabAppImplicitCore___lambda__11___closed__2; +x_2 = l_Lean_PrettyPrinter_Delaborator_delabDo___closed__2; +x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Delaborator_whenPPOption), 9, 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_Delaborator_delabDo(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; lean_object* x_9; lean_object* x_10; -x_8 = l_Lean_PrettyPrinter_Delaborator_delabAppImplicitCore___lambda__11___closed__2; -x_9 = l_Lean_PrettyPrinter_Delaborator_delabDo___closed__2; -x_10 = l_Lean_PrettyPrinter_Delaborator_whenPPOption(x_8, x_9, x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Lean_PrettyPrinter_Delaborator_useAppExplicit___closed__1; +x_9 = l_Lean_PrettyPrinter_Delaborator_delabDo___closed__3; +x_10 = l_Lean_PrettyPrinter_Delaborator_whenNotPPOption(x_8, x_9, x_1, x_2, x_3, x_4, x_5, x_6, x_7); return x_10; } } @@ -45078,3626 +45283,456 @@ x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); return x_6; } } -static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1() { +LEAN_EXPORT uint8_t l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__1(lean_object* x_1) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Name", 4, 4); -return x_1; +uint8_t x_2; +x_2 = 0; +return x_2; } } -static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__2() { +static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("anonymous", 9, 9); +x_1 = lean_mk_string_unchecked("quotedName", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__3() { +static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("mkStr1", 6, 6); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; +x_2 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__3; +x_3 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__4; +x_4 = l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__1; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; } } -static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__4() { +static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__3() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("str", 3, 3); +x_1 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__1___boxed), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__5() { +static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__4() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("num", 3, 3); +x_1 = lean_mk_string_unchecked("`", 1, 1); return x_1; } } -static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__6() { +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("mkStr2", 6, 6); -return x_1; +lean_object* x_9; +x_9 = l_Lean_Expr_name_x3f(x_1); +if (lean_obj_tag(x_9) == 0) +{ +lean_object* x_10; +x_10 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); +return x_10; +} +else +{ +lean_object* x_11; uint8_t x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_11 = lean_ctor_get(x_9, 0); +lean_inc(x_11); +lean_dec(x_9); +x_12 = 1; +x_13 = l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__3; +x_14 = l_Lean_Name_toString(x_11, x_12, x_13); +x_15 = l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__4; +x_16 = lean_string_append(x_15, x_14); +lean_dec(x_14); +x_17 = l_Lean_PrettyPrinter_Delaborator_delabOfScientific___lambda__1___closed__2; +x_18 = lean_string_append(x_16, x_17); +x_19 = lean_box(2); +x_20 = l_Lean_Syntax_mkNameLit(x_18, x_19); +x_21 = lean_box(0); +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_array_mk(x_22); +x_24 = l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__2; +x_25 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_25, 0, x_19); +lean_ctor_set(x_25, 1, x_24); +lean_ctor_set(x_25, 2, x_23); +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_8); +return x_26; +} } } -static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__7() { +static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("mkStr3", 6, 6); +x_1 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___boxed), 8, 0); return x_1; } } -static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__8() { +static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("mkStr4", 6, 6); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_PrettyPrinter_Delaborator_delabAppExplicitCore___closed__1; +x_2 = l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___closed__1; +x_3 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_PrettyPrinter_Delaborator_delabMVarAux___spec__1___rarg), 9, 2); +lean_closure_set(x_3, 0, x_1); +lean_closure_set(x_3, 1, x_2); +return x_3; } } -static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__9() { +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabNameMkStr(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("mkStr5", 6, 6); -return x_1; +lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_8 = l_Lean_PrettyPrinter_Delaborator_delabAppImplicitCore___lambda__11___closed__2; +x_9 = l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___closed__2; +x_10 = l_Lean_PrettyPrinter_Delaborator_whenPPOption(x_8, x_9, x_1, x_2, x_3, x_4, x_5, x_6, x_7); +return x_10; } } -static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__10() { +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__1___boxed(lean_object* x_1) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("mkStr6", 6, 6); -return x_1; +uint8_t x_2; lean_object* x_3; +x_2 = l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__1(x_1); +lean_dec(x_1); +x_3 = lean_box(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +x_9 = l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_9; } } -static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__11() { +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("mkStr7", 6, 6); +x_1 = lean_mk_string_unchecked("Name", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__12() { +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__2() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("mkStr8", 6, 6); +x_1 = lean_mk_string_unchecked("str", 3, 3); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_reifyName(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__3() { _start: { -switch (lean_obj_tag(x_1)) { -case 4: -{ -lean_object* x_9; -x_9 = lean_ctor_get(x_1, 0); -lean_inc(x_9); -lean_dec(x_1); -if (lean_obj_tag(x_9) == 1) -{ -lean_object* x_10; -x_10 = lean_ctor_get(x_9, 0); -lean_inc(x_10); -if (lean_obj_tag(x_10) == 1) -{ -lean_object* x_11; -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -if (lean_obj_tag(x_11) == 1) -{ -lean_object* x_12; -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); -if (lean_obj_tag(x_12) == 0) -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; -x_13 = lean_ctor_get(x_9, 1); -lean_inc(x_13); -lean_dec(x_9); -x_14 = lean_ctor_get(x_10, 1); -lean_inc(x_14); -lean_dec(x_10); -x_15 = lean_ctor_get(x_11, 1); -lean_inc(x_15); -lean_dec(x_11); -x_16 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_17 = lean_string_dec_eq(x_15, x_16); -lean_dec(x_15); -if (x_17 == 0) -{ -lean_object* x_18; -lean_dec(x_14); -lean_dec(x_13); -x_18 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_18; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabApp__1___closed__1; +x_2 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__1; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__2; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; } -else -{ -lean_object* x_19; uint8_t x_20; -x_19 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_20 = lean_string_dec_eq(x_14, x_19); -lean_dec(x_14); -if (x_20 == 0) -{ -lean_object* x_21; -lean_dec(x_13); -x_21 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_21; } -else -{ -lean_object* x_22; uint8_t x_23; -x_22 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__2; -x_23 = lean_string_dec_eq(x_13, x_22); -lean_dec(x_13); -if (x_23 == 0) +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__4() { +_start: { -lean_object* x_24; -x_24 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_24; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("delabNameMkStr", 14, 14); +return x_1; } -else +} +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__5() { +_start: { -lean_object* x_25; lean_object* x_26; -x_25 = lean_box(0); -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_26, 1, x_8); -return x_26; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; +x_2 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabFVar__1___closed__3; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabFVar__1___closed__4; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__4; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; } } +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Delaborator_delabNameMkStr), 7, 0); +return x_1; } } -else +LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1(lean_object* x_1) { +_start: { -lean_object* x_27; -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -x_27 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_27; +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabFVar__1___closed__7; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__3; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__5; +x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__6; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; } } -else +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__2___closed__1() { +_start: { -lean_object* x_28; -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -x_28 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_28; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mkStr1", 6, 6); +return x_1; } } -else +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__2___closed__2() { +_start: { -lean_object* x_29; -lean_dec(x_10); -lean_dec(x_9); -x_29 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_29; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabApp__1___closed__1; +x_2 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__1; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__2___closed__1; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; } } -else +LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__2(lean_object* x_1) { +_start: { -lean_object* x_30; -lean_dec(x_9); -x_30 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_30; +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabFVar__1___closed__7; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__2___closed__2; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__5; +x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__6; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; } } -case 5: -{ -lean_object* x_31; -x_31 = lean_ctor_get(x_1, 0); -lean_inc(x_31); -switch (lean_obj_tag(x_31)) { -case 4: -{ -lean_object* x_32; -x_32 = lean_ctor_get(x_31, 0); -lean_inc(x_32); -lean_dec(x_31); -if (lean_obj_tag(x_32) == 1) -{ -lean_object* x_33; -x_33 = lean_ctor_get(x_32, 0); -lean_inc(x_33); -if (lean_obj_tag(x_33) == 1) -{ -lean_object* x_34; -x_34 = lean_ctor_get(x_33, 0); -lean_inc(x_34); -if (lean_obj_tag(x_34) == 1) +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__3___closed__1() { +_start: { -lean_object* x_35; -x_35 = lean_ctor_get(x_34, 0); -lean_inc(x_35); -if (lean_obj_tag(x_35) == 0) +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mkStr2", 6, 6); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__3___closed__2() { +_start: { -lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; -x_36 = lean_ctor_get(x_1, 1); -lean_inc(x_36); -lean_dec(x_1); -x_37 = lean_ctor_get(x_32, 1); -lean_inc(x_37); -lean_dec(x_32); -x_38 = lean_ctor_get(x_33, 1); -lean_inc(x_38); -lean_dec(x_33); -x_39 = lean_ctor_get(x_34, 1); -lean_inc(x_39); -lean_dec(x_34); -x_40 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_41 = lean_string_dec_eq(x_39, x_40); -lean_dec(x_39); -if (x_41 == 0) +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabApp__1___closed__1; +x_2 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__1; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__3___closed__1; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__3(lean_object* x_1) { +_start: { -lean_object* x_42; -lean_dec(x_38); -lean_dec(x_37); -lean_dec(x_36); -x_42 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_42; +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabFVar__1___closed__7; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__3___closed__2; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__5; +x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__6; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; } -else +} +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__4___closed__1() { +_start: { -lean_object* x_43; uint8_t x_44; -x_43 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_44 = lean_string_dec_eq(x_38, x_43); -lean_dec(x_38); -if (x_44 == 0) +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mkStr3", 6, 6); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__4___closed__2() { +_start: { -lean_object* x_45; -lean_dec(x_37); -lean_dec(x_36); -x_45 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_45; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabApp__1___closed__1; +x_2 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__1; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__4___closed__1; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; } -else +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__4(lean_object* x_1) { +_start: { -lean_object* x_46; uint8_t x_47; -x_46 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__3; -x_47 = lean_string_dec_eq(x_37, x_46); -lean_dec(x_37); -if (x_47 == 0) +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabFVar__1___closed__7; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__4___closed__2; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__5; +x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__6; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__5___closed__1() { +_start: { -lean_object* x_48; -lean_dec(x_36); -x_48 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_48; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mkStr4", 6, 6); +return x_1; } -else +} +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__5___closed__2() { +_start: { -if (lean_obj_tag(x_36) == 9) +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabApp__1___closed__1; +x_2 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__1; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__5___closed__1; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__5(lean_object* x_1) { +_start: { -lean_object* x_49; -x_49 = lean_ctor_get(x_36, 0); -lean_inc(x_49); -lean_dec(x_36); -if (lean_obj_tag(x_49) == 0) +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabFVar__1___closed__7; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__5___closed__2; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__5; +x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__6; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__6___closed__1() { +_start: { -lean_object* x_50; -lean_dec(x_49); -x_50 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_50; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mkStr5", 6, 6); +return x_1; } -else +} +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__6___closed__2() { +_start: { -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; -x_51 = lean_ctor_get(x_49, 0); -lean_inc(x_51); -lean_dec(x_49); -x_52 = lean_box(0); -x_53 = l_Lean_Name_str___override(x_52, x_51); -x_54 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_54, 0, x_53); -lean_ctor_set(x_54, 1, x_8); -return x_54; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabApp__1___closed__1; +x_2 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__1; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__6___closed__1; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; } } -else +LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__6(lean_object* x_1) { +_start: { -lean_object* x_55; -lean_dec(x_36); -x_55 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_55; +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabFVar__1___closed__7; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__6___closed__2; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__5; +x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__6; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; } } +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__7___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mkStr6", 6, 6); +return x_1; +} } +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__7___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabApp__1___closed__1; +x_2 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__1; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__7___closed__1; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; } } -else +LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__7(lean_object* x_1) { +_start: { -lean_object* x_56; -lean_dec(x_35); -lean_dec(x_34); -lean_dec(x_33); -lean_dec(x_32); -lean_dec(x_1); -x_56 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_56; +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabFVar__1___closed__7; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__7___closed__2; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__5; +x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__6; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; } } -else +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__8___closed__1() { +_start: { -lean_object* x_57; -lean_dec(x_34); -lean_dec(x_33); -lean_dec(x_32); -lean_dec(x_1); -x_57 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_57; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mkStr7", 6, 6); +return x_1; } } -else +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__8___closed__2() { +_start: { -lean_object* x_58; -lean_dec(x_33); -lean_dec(x_32); -lean_dec(x_1); -x_58 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_58; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabApp__1___closed__1; +x_2 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__1; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__8___closed__1; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; } } -else +LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__8(lean_object* x_1) { +_start: { -lean_object* x_59; -lean_dec(x_32); -lean_dec(x_1); -x_59 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_59; +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabFVar__1___closed__7; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__8___closed__2; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__5; +x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__6; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; } } -case 5: -{ -lean_object* x_60; -x_60 = lean_ctor_get(x_31, 0); -lean_inc(x_60); -switch (lean_obj_tag(x_60)) { -case 4: -{ -lean_object* x_61; -x_61 = lean_ctor_get(x_60, 0); -lean_inc(x_61); -lean_dec(x_60); -if (lean_obj_tag(x_61) == 1) -{ -lean_object* x_62; -x_62 = lean_ctor_get(x_61, 0); -lean_inc(x_62); -if (lean_obj_tag(x_62) == 1) -{ -lean_object* x_63; -x_63 = lean_ctor_get(x_62, 0); -lean_inc(x_63); -if (lean_obj_tag(x_63) == 1) -{ -lean_object* x_64; -x_64 = lean_ctor_get(x_63, 0); -lean_inc(x_64); -if (lean_obj_tag(x_64) == 0) -{ -lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; uint8_t x_71; -x_65 = lean_ctor_get(x_1, 1); -lean_inc(x_65); -lean_dec(x_1); -x_66 = lean_ctor_get(x_31, 1); -lean_inc(x_66); -lean_dec(x_31); -x_67 = lean_ctor_get(x_61, 1); -lean_inc(x_67); -lean_dec(x_61); -x_68 = lean_ctor_get(x_62, 1); -lean_inc(x_68); -lean_dec(x_62); -x_69 = lean_ctor_get(x_63, 1); -lean_inc(x_69); -lean_dec(x_63); -x_70 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_71 = lean_string_dec_eq(x_69, x_70); -lean_dec(x_69); -if (x_71 == 0) -{ -lean_object* x_72; -lean_dec(x_68); -lean_dec(x_67); -lean_dec(x_66); -lean_dec(x_65); -x_72 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_72; -} -else -{ -lean_object* x_73; uint8_t x_74; -x_73 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_74 = lean_string_dec_eq(x_68, x_73); -lean_dec(x_68); -if (x_74 == 0) -{ -lean_object* x_75; -lean_dec(x_67); -lean_dec(x_66); -lean_dec(x_65); -x_75 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_75; -} -else -{ -lean_object* x_76; uint8_t x_77; -x_76 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__4; -x_77 = lean_string_dec_eq(x_67, x_76); -if (x_77 == 0) -{ -lean_object* x_78; uint8_t x_79; -x_78 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__5; -x_79 = lean_string_dec_eq(x_67, x_78); -if (x_79 == 0) -{ -lean_object* x_80; uint8_t x_81; -x_80 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__6; -x_81 = lean_string_dec_eq(x_67, x_80); -lean_dec(x_67); -if (x_81 == 0) -{ -lean_object* x_82; -lean_dec(x_66); -lean_dec(x_65); -x_82 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_82; -} -else -{ -if (lean_obj_tag(x_66) == 9) -{ -lean_object* x_83; -x_83 = lean_ctor_get(x_66, 0); -lean_inc(x_83); -lean_dec(x_66); -if (lean_obj_tag(x_83) == 0) -{ -lean_object* x_84; -lean_dec(x_83); -lean_dec(x_65); -x_84 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_84; -} -else -{ -if (lean_obj_tag(x_65) == 9) -{ -lean_object* x_85; -x_85 = lean_ctor_get(x_65, 0); -lean_inc(x_85); -lean_dec(x_65); -if (lean_obj_tag(x_85) == 0) -{ -lean_object* x_86; -lean_dec(x_85); -lean_dec(x_83); -x_86 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_86; -} -else -{ -lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; -x_87 = lean_ctor_get(x_83, 0); -lean_inc(x_87); -lean_dec(x_83); -x_88 = lean_ctor_get(x_85, 0); -lean_inc(x_88); -lean_dec(x_85); -x_89 = l_Lean_Name_mkStr2(x_87, x_88); -x_90 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_90, 0, x_89); -lean_ctor_set(x_90, 1, x_8); -return x_90; -} -} -else -{ -lean_object* x_91; -lean_dec(x_83); -lean_dec(x_65); -x_91 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_91; -} -} -} -else -{ -lean_object* x_92; -lean_dec(x_66); -lean_dec(x_65); -x_92 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_92; -} -} -} -else -{ -lean_dec(x_67); -if (lean_obj_tag(x_65) == 9) -{ -lean_object* x_93; -x_93 = lean_ctor_get(x_65, 0); -lean_inc(x_93); -lean_dec(x_65); -if (lean_obj_tag(x_93) == 0) -{ -lean_object* x_94; lean_object* x_95; -x_94 = lean_ctor_get(x_93, 0); -lean_inc(x_94); -lean_dec(x_93); -x_95 = l_Lean_PrettyPrinter_Delaborator_reifyName(x_66, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_95) == 0) -{ -uint8_t x_96; -x_96 = !lean_is_exclusive(x_95); -if (x_96 == 0) -{ -lean_object* x_97; lean_object* x_98; -x_97 = lean_ctor_get(x_95, 0); -x_98 = l_Lean_Name_num___override(x_97, x_94); -lean_ctor_set(x_95, 0, x_98); -return x_95; -} -else -{ -lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; -x_99 = lean_ctor_get(x_95, 0); -x_100 = lean_ctor_get(x_95, 1); -lean_inc(x_100); -lean_inc(x_99); -lean_dec(x_95); -x_101 = l_Lean_Name_num___override(x_99, x_94); -x_102 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_102, 0, x_101); -lean_ctor_set(x_102, 1, x_100); -return x_102; -} -} -else -{ -uint8_t x_103; -lean_dec(x_94); -x_103 = !lean_is_exclusive(x_95); -if (x_103 == 0) -{ -return x_95; -} -else -{ -lean_object* x_104; lean_object* x_105; lean_object* x_106; -x_104 = lean_ctor_get(x_95, 0); -x_105 = lean_ctor_get(x_95, 1); -lean_inc(x_105); -lean_inc(x_104); -lean_dec(x_95); -x_106 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_106, 0, x_104); -lean_ctor_set(x_106, 1, x_105); -return x_106; -} -} -} -else -{ -lean_object* x_107; -lean_dec(x_93); -lean_dec(x_66); -x_107 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_107; -} -} -else -{ -lean_object* x_108; -lean_dec(x_66); -lean_dec(x_65); -x_108 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_108; -} -} -} -else -{ -lean_dec(x_67); -if (lean_obj_tag(x_65) == 9) -{ -lean_object* x_109; -x_109 = lean_ctor_get(x_65, 0); -lean_inc(x_109); -lean_dec(x_65); -if (lean_obj_tag(x_109) == 0) -{ -lean_object* x_110; -lean_dec(x_109); -lean_dec(x_66); -x_110 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_110; -} -else -{ -lean_object* x_111; lean_object* x_112; -x_111 = lean_ctor_get(x_109, 0); -lean_inc(x_111); -lean_dec(x_109); -x_112 = l_Lean_PrettyPrinter_Delaborator_reifyName(x_66, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_112) == 0) -{ -uint8_t x_113; -x_113 = !lean_is_exclusive(x_112); -if (x_113 == 0) -{ -lean_object* x_114; lean_object* x_115; -x_114 = lean_ctor_get(x_112, 0); -x_115 = l_Lean_Name_str___override(x_114, x_111); -lean_ctor_set(x_112, 0, x_115); -return x_112; -} -else -{ -lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; -x_116 = lean_ctor_get(x_112, 0); -x_117 = lean_ctor_get(x_112, 1); -lean_inc(x_117); -lean_inc(x_116); -lean_dec(x_112); -x_118 = l_Lean_Name_str___override(x_116, x_111); -x_119 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_119, 0, x_118); -lean_ctor_set(x_119, 1, x_117); -return x_119; -} -} -else -{ -uint8_t x_120; -lean_dec(x_111); -x_120 = !lean_is_exclusive(x_112); -if (x_120 == 0) -{ -return x_112; -} -else -{ -lean_object* x_121; lean_object* x_122; lean_object* x_123; -x_121 = lean_ctor_get(x_112, 0); -x_122 = lean_ctor_get(x_112, 1); -lean_inc(x_122); -lean_inc(x_121); -lean_dec(x_112); -x_123 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_123, 0, x_121); -lean_ctor_set(x_123, 1, x_122); -return x_123; -} -} -} -} -else -{ -lean_object* x_124; -lean_dec(x_66); -lean_dec(x_65); -x_124 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_124; -} -} -} -} -} -else -{ -lean_object* x_125; -lean_dec(x_64); -lean_dec(x_63); -lean_dec(x_62); -lean_dec(x_61); -lean_dec(x_31); -lean_dec(x_1); -x_125 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_125; -} -} -else -{ -lean_object* x_126; -lean_dec(x_63); -lean_dec(x_62); -lean_dec(x_61); -lean_dec(x_31); -lean_dec(x_1); -x_126 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_126; -} -} -else -{ -lean_object* x_127; -lean_dec(x_62); -lean_dec(x_61); -lean_dec(x_31); -lean_dec(x_1); -x_127 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_127; -} -} -else -{ -lean_object* x_128; -lean_dec(x_61); -lean_dec(x_31); -lean_dec(x_1); -x_128 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_128; -} -} -case 5: -{ -lean_object* x_129; -x_129 = lean_ctor_get(x_60, 0); -lean_inc(x_129); -switch (lean_obj_tag(x_129)) { -case 4: -{ -lean_object* x_130; -x_130 = lean_ctor_get(x_129, 0); -lean_inc(x_130); -lean_dec(x_129); -if (lean_obj_tag(x_130) == 1) -{ -lean_object* x_131; -x_131 = lean_ctor_get(x_130, 0); -lean_inc(x_131); -if (lean_obj_tag(x_131) == 1) -{ -lean_object* x_132; -x_132 = lean_ctor_get(x_131, 0); -lean_inc(x_132); -if (lean_obj_tag(x_132) == 1) -{ -lean_object* x_133; -x_133 = lean_ctor_get(x_132, 0); -lean_inc(x_133); -if (lean_obj_tag(x_133) == 0) -{ -lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; uint8_t x_141; -x_134 = lean_ctor_get(x_1, 1); -lean_inc(x_134); -lean_dec(x_1); -x_135 = lean_ctor_get(x_31, 1); -lean_inc(x_135); -lean_dec(x_31); -x_136 = lean_ctor_get(x_60, 1); -lean_inc(x_136); -lean_dec(x_60); -x_137 = lean_ctor_get(x_130, 1); -lean_inc(x_137); -lean_dec(x_130); -x_138 = lean_ctor_get(x_131, 1); -lean_inc(x_138); -lean_dec(x_131); -x_139 = lean_ctor_get(x_132, 1); -lean_inc(x_139); -lean_dec(x_132); -x_140 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_141 = lean_string_dec_eq(x_139, x_140); -lean_dec(x_139); -if (x_141 == 0) -{ -lean_object* x_142; -lean_dec(x_138); -lean_dec(x_137); -lean_dec(x_136); -lean_dec(x_135); -lean_dec(x_134); -x_142 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_142; -} -else -{ -lean_object* x_143; uint8_t x_144; -x_143 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_144 = lean_string_dec_eq(x_138, x_143); -lean_dec(x_138); -if (x_144 == 0) -{ -lean_object* x_145; -lean_dec(x_137); -lean_dec(x_136); -lean_dec(x_135); -lean_dec(x_134); -x_145 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_145; -} -else -{ -lean_object* x_146; uint8_t x_147; -x_146 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__7; -x_147 = lean_string_dec_eq(x_137, x_146); -lean_dec(x_137); -if (x_147 == 0) -{ -lean_object* x_148; -lean_dec(x_136); -lean_dec(x_135); -lean_dec(x_134); -x_148 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_148; -} -else -{ -if (lean_obj_tag(x_136) == 9) -{ -lean_object* x_149; -x_149 = lean_ctor_get(x_136, 0); -lean_inc(x_149); -lean_dec(x_136); -if (lean_obj_tag(x_149) == 0) -{ -lean_object* x_150; -lean_dec(x_149); -lean_dec(x_135); -lean_dec(x_134); -x_150 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_150; -} -else -{ -if (lean_obj_tag(x_135) == 9) -{ -lean_object* x_151; -x_151 = lean_ctor_get(x_135, 0); -lean_inc(x_151); -lean_dec(x_135); -if (lean_obj_tag(x_151) == 0) -{ -lean_object* x_152; -lean_dec(x_151); -lean_dec(x_149); -lean_dec(x_134); -x_152 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_152; -} -else -{ -if (lean_obj_tag(x_134) == 9) -{ -lean_object* x_153; -x_153 = lean_ctor_get(x_134, 0); -lean_inc(x_153); -lean_dec(x_134); -if (lean_obj_tag(x_153) == 0) -{ -lean_object* x_154; -lean_dec(x_153); -lean_dec(x_151); -lean_dec(x_149); -x_154 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_154; -} -else -{ -lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; -x_155 = lean_ctor_get(x_149, 0); -lean_inc(x_155); -lean_dec(x_149); -x_156 = lean_ctor_get(x_151, 0); -lean_inc(x_156); -lean_dec(x_151); -x_157 = lean_ctor_get(x_153, 0); -lean_inc(x_157); -lean_dec(x_153); -x_158 = l_Lean_Name_mkStr3(x_155, x_156, x_157); -x_159 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_159, 0, x_158); -lean_ctor_set(x_159, 1, x_8); -return x_159; -} -} -else -{ -lean_object* x_160; -lean_dec(x_151); -lean_dec(x_149); -lean_dec(x_134); -x_160 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_160; -} -} -} -else -{ -lean_object* x_161; -lean_dec(x_149); -lean_dec(x_135); -lean_dec(x_134); -x_161 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_161; -} -} -} -else -{ -lean_object* x_162; -lean_dec(x_136); -lean_dec(x_135); -lean_dec(x_134); -x_162 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_162; -} -} -} -} -} -else -{ -lean_object* x_163; -lean_dec(x_133); -lean_dec(x_132); -lean_dec(x_131); -lean_dec(x_130); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_163 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_163; -} -} -else -{ -lean_object* x_164; -lean_dec(x_132); -lean_dec(x_131); -lean_dec(x_130); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_164 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_164; -} -} -else -{ -lean_object* x_165; -lean_dec(x_131); -lean_dec(x_130); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_165 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_165; -} -} -else -{ -lean_object* x_166; -lean_dec(x_130); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_166 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_166; -} -} -case 5: -{ -lean_object* x_167; -x_167 = lean_ctor_get(x_129, 0); -lean_inc(x_167); -switch (lean_obj_tag(x_167)) { -case 4: -{ -lean_object* x_168; -x_168 = lean_ctor_get(x_167, 0); -lean_inc(x_168); -lean_dec(x_167); -if (lean_obj_tag(x_168) == 1) -{ -lean_object* x_169; -x_169 = lean_ctor_get(x_168, 0); -lean_inc(x_169); -if (lean_obj_tag(x_169) == 1) -{ -lean_object* x_170; -x_170 = lean_ctor_get(x_169, 0); -lean_inc(x_170); -if (lean_obj_tag(x_170) == 1) -{ -lean_object* x_171; -x_171 = lean_ctor_get(x_170, 0); -lean_inc(x_171); -if (lean_obj_tag(x_171) == 0) -{ -lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; uint8_t x_180; -x_172 = lean_ctor_get(x_1, 1); -lean_inc(x_172); -lean_dec(x_1); -x_173 = lean_ctor_get(x_31, 1); -lean_inc(x_173); -lean_dec(x_31); -x_174 = lean_ctor_get(x_60, 1); -lean_inc(x_174); -lean_dec(x_60); -x_175 = lean_ctor_get(x_129, 1); -lean_inc(x_175); -lean_dec(x_129); -x_176 = lean_ctor_get(x_168, 1); -lean_inc(x_176); -lean_dec(x_168); -x_177 = lean_ctor_get(x_169, 1); -lean_inc(x_177); -lean_dec(x_169); -x_178 = lean_ctor_get(x_170, 1); -lean_inc(x_178); -lean_dec(x_170); -x_179 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_180 = lean_string_dec_eq(x_178, x_179); -lean_dec(x_178); -if (x_180 == 0) -{ -lean_object* x_181; -lean_dec(x_177); -lean_dec(x_176); -lean_dec(x_175); -lean_dec(x_174); -lean_dec(x_173); -lean_dec(x_172); -x_181 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_181; -} -else -{ -lean_object* x_182; uint8_t x_183; -x_182 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_183 = lean_string_dec_eq(x_177, x_182); -lean_dec(x_177); -if (x_183 == 0) -{ -lean_object* x_184; -lean_dec(x_176); -lean_dec(x_175); -lean_dec(x_174); -lean_dec(x_173); -lean_dec(x_172); -x_184 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_184; -} -else -{ -lean_object* x_185; uint8_t x_186; -x_185 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__8; -x_186 = lean_string_dec_eq(x_176, x_185); -lean_dec(x_176); -if (x_186 == 0) -{ -lean_object* x_187; -lean_dec(x_175); -lean_dec(x_174); -lean_dec(x_173); -lean_dec(x_172); -x_187 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_187; -} -else -{ -if (lean_obj_tag(x_175) == 9) -{ -lean_object* x_188; -x_188 = lean_ctor_get(x_175, 0); -lean_inc(x_188); -lean_dec(x_175); -if (lean_obj_tag(x_188) == 0) -{ -lean_object* x_189; -lean_dec(x_188); -lean_dec(x_174); -lean_dec(x_173); -lean_dec(x_172); -x_189 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_189; -} -else -{ -if (lean_obj_tag(x_174) == 9) -{ -lean_object* x_190; -x_190 = lean_ctor_get(x_174, 0); -lean_inc(x_190); -lean_dec(x_174); -if (lean_obj_tag(x_190) == 0) -{ -lean_object* x_191; -lean_dec(x_190); -lean_dec(x_188); -lean_dec(x_173); -lean_dec(x_172); -x_191 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_191; -} -else -{ -if (lean_obj_tag(x_173) == 9) -{ -lean_object* x_192; -x_192 = lean_ctor_get(x_173, 0); -lean_inc(x_192); -lean_dec(x_173); -if (lean_obj_tag(x_192) == 0) -{ -lean_object* x_193; -lean_dec(x_192); -lean_dec(x_190); -lean_dec(x_188); -lean_dec(x_172); -x_193 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_193; -} -else -{ -if (lean_obj_tag(x_172) == 9) -{ -lean_object* x_194; -x_194 = lean_ctor_get(x_172, 0); -lean_inc(x_194); -lean_dec(x_172); -if (lean_obj_tag(x_194) == 0) -{ -lean_object* x_195; -lean_dec(x_194); -lean_dec(x_192); -lean_dec(x_190); -lean_dec(x_188); -x_195 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_195; -} -else -{ -lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; -x_196 = lean_ctor_get(x_188, 0); -lean_inc(x_196); -lean_dec(x_188); -x_197 = lean_ctor_get(x_190, 0); -lean_inc(x_197); -lean_dec(x_190); -x_198 = lean_ctor_get(x_192, 0); -lean_inc(x_198); -lean_dec(x_192); -x_199 = lean_ctor_get(x_194, 0); -lean_inc(x_199); -lean_dec(x_194); -x_200 = l_Lean_Name_mkStr4(x_196, x_197, x_198, x_199); -x_201 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_201, 0, x_200); -lean_ctor_set(x_201, 1, x_8); -return x_201; -} -} -else -{ -lean_object* x_202; -lean_dec(x_192); -lean_dec(x_190); -lean_dec(x_188); -lean_dec(x_172); -x_202 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_202; -} -} -} -else -{ -lean_object* x_203; -lean_dec(x_190); -lean_dec(x_188); -lean_dec(x_173); -lean_dec(x_172); -x_203 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_203; -} -} -} -else -{ -lean_object* x_204; -lean_dec(x_188); -lean_dec(x_174); -lean_dec(x_173); -lean_dec(x_172); -x_204 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_204; -} -} -} -else -{ -lean_object* x_205; -lean_dec(x_175); -lean_dec(x_174); -lean_dec(x_173); -lean_dec(x_172); -x_205 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_205; -} -} -} -} -} -else -{ -lean_object* x_206; -lean_dec(x_171); -lean_dec(x_170); -lean_dec(x_169); -lean_dec(x_168); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_206 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_206; -} -} -else -{ -lean_object* x_207; -lean_dec(x_170); -lean_dec(x_169); -lean_dec(x_168); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_207 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_207; -} -} -else -{ -lean_object* x_208; -lean_dec(x_169); -lean_dec(x_168); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_208 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_208; -} -} -else -{ -lean_object* x_209; -lean_dec(x_168); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_209 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_209; -} -} -case 5: -{ -lean_object* x_210; -x_210 = lean_ctor_get(x_167, 0); -lean_inc(x_210); -switch (lean_obj_tag(x_210)) { -case 4: -{ -lean_object* x_211; -x_211 = lean_ctor_get(x_210, 0); -lean_inc(x_211); -lean_dec(x_210); -if (lean_obj_tag(x_211) == 1) -{ -lean_object* x_212; -x_212 = lean_ctor_get(x_211, 0); -lean_inc(x_212); -if (lean_obj_tag(x_212) == 1) -{ -lean_object* x_213; -x_213 = lean_ctor_get(x_212, 0); -lean_inc(x_213); -if (lean_obj_tag(x_213) == 1) -{ -lean_object* x_214; -x_214 = lean_ctor_get(x_213, 0); -lean_inc(x_214); -if (lean_obj_tag(x_214) == 0) -{ -lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; uint8_t x_224; -x_215 = lean_ctor_get(x_1, 1); -lean_inc(x_215); -lean_dec(x_1); -x_216 = lean_ctor_get(x_31, 1); -lean_inc(x_216); -lean_dec(x_31); -x_217 = lean_ctor_get(x_60, 1); -lean_inc(x_217); -lean_dec(x_60); -x_218 = lean_ctor_get(x_129, 1); -lean_inc(x_218); -lean_dec(x_129); -x_219 = lean_ctor_get(x_167, 1); -lean_inc(x_219); -lean_dec(x_167); -x_220 = lean_ctor_get(x_211, 1); -lean_inc(x_220); -lean_dec(x_211); -x_221 = lean_ctor_get(x_212, 1); -lean_inc(x_221); -lean_dec(x_212); -x_222 = lean_ctor_get(x_213, 1); -lean_inc(x_222); -lean_dec(x_213); -x_223 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_224 = lean_string_dec_eq(x_222, x_223); -lean_dec(x_222); -if (x_224 == 0) -{ -lean_object* x_225; -lean_dec(x_221); -lean_dec(x_220); -lean_dec(x_219); -lean_dec(x_218); -lean_dec(x_217); -lean_dec(x_216); -lean_dec(x_215); -x_225 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_225; -} -else -{ -lean_object* x_226; uint8_t x_227; -x_226 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_227 = lean_string_dec_eq(x_221, x_226); -lean_dec(x_221); -if (x_227 == 0) -{ -lean_object* x_228; -lean_dec(x_220); -lean_dec(x_219); -lean_dec(x_218); -lean_dec(x_217); -lean_dec(x_216); -lean_dec(x_215); -x_228 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_228; -} -else -{ -lean_object* x_229; uint8_t x_230; -x_229 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__9; -x_230 = lean_string_dec_eq(x_220, x_229); -lean_dec(x_220); -if (x_230 == 0) -{ -lean_object* x_231; -lean_dec(x_219); -lean_dec(x_218); -lean_dec(x_217); -lean_dec(x_216); -lean_dec(x_215); -x_231 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_231; -} -else -{ -if (lean_obj_tag(x_219) == 9) -{ -lean_object* x_232; -x_232 = lean_ctor_get(x_219, 0); -lean_inc(x_232); -lean_dec(x_219); -if (lean_obj_tag(x_232) == 0) -{ -lean_object* x_233; -lean_dec(x_232); -lean_dec(x_218); -lean_dec(x_217); -lean_dec(x_216); -lean_dec(x_215); -x_233 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_233; -} -else -{ -if (lean_obj_tag(x_218) == 9) -{ -lean_object* x_234; -x_234 = lean_ctor_get(x_218, 0); -lean_inc(x_234); -lean_dec(x_218); -if (lean_obj_tag(x_234) == 0) -{ -lean_object* x_235; -lean_dec(x_234); -lean_dec(x_232); -lean_dec(x_217); -lean_dec(x_216); -lean_dec(x_215); -x_235 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_235; -} -else -{ -if (lean_obj_tag(x_217) == 9) -{ -lean_object* x_236; -x_236 = lean_ctor_get(x_217, 0); -lean_inc(x_236); -lean_dec(x_217); -if (lean_obj_tag(x_236) == 0) -{ -lean_object* x_237; -lean_dec(x_236); -lean_dec(x_234); -lean_dec(x_232); -lean_dec(x_216); -lean_dec(x_215); -x_237 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_237; -} -else -{ -if (lean_obj_tag(x_216) == 9) -{ -lean_object* x_238; -x_238 = lean_ctor_get(x_216, 0); -lean_inc(x_238); -lean_dec(x_216); -if (lean_obj_tag(x_238) == 0) -{ -lean_object* x_239; -lean_dec(x_238); -lean_dec(x_236); -lean_dec(x_234); -lean_dec(x_232); -lean_dec(x_215); -x_239 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_239; -} -else -{ -if (lean_obj_tag(x_215) == 9) -{ -lean_object* x_240; -x_240 = lean_ctor_get(x_215, 0); -lean_inc(x_240); -lean_dec(x_215); -if (lean_obj_tag(x_240) == 0) -{ -lean_object* x_241; -lean_dec(x_240); -lean_dec(x_238); -lean_dec(x_236); -lean_dec(x_234); -lean_dec(x_232); -x_241 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_241; -} -else -{ -lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; -x_242 = lean_ctor_get(x_232, 0); -lean_inc(x_242); -lean_dec(x_232); -x_243 = lean_ctor_get(x_234, 0); -lean_inc(x_243); -lean_dec(x_234); -x_244 = lean_ctor_get(x_236, 0); -lean_inc(x_244); -lean_dec(x_236); -x_245 = lean_ctor_get(x_238, 0); -lean_inc(x_245); -lean_dec(x_238); -x_246 = lean_ctor_get(x_240, 0); -lean_inc(x_246); -lean_dec(x_240); -x_247 = l_Lean_Name_mkStr5(x_242, x_243, x_244, x_245, x_246); -x_248 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_248, 0, x_247); -lean_ctor_set(x_248, 1, x_8); -return x_248; -} -} -else -{ -lean_object* x_249; -lean_dec(x_238); -lean_dec(x_236); -lean_dec(x_234); -lean_dec(x_232); -lean_dec(x_215); -x_249 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_249; -} -} -} -else -{ -lean_object* x_250; -lean_dec(x_236); -lean_dec(x_234); -lean_dec(x_232); -lean_dec(x_216); -lean_dec(x_215); -x_250 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_250; -} -} -} -else -{ -lean_object* x_251; -lean_dec(x_234); -lean_dec(x_232); -lean_dec(x_217); -lean_dec(x_216); -lean_dec(x_215); -x_251 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_251; -} -} -} -else -{ -lean_object* x_252; -lean_dec(x_232); -lean_dec(x_218); -lean_dec(x_217); -lean_dec(x_216); -lean_dec(x_215); -x_252 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_252; -} -} -} -else -{ -lean_object* x_253; -lean_dec(x_219); -lean_dec(x_218); -lean_dec(x_217); -lean_dec(x_216); -lean_dec(x_215); -x_253 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_253; -} -} -} -} -} -else -{ -lean_object* x_254; -lean_dec(x_214); -lean_dec(x_213); -lean_dec(x_212); -lean_dec(x_211); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_254 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_254; -} -} -else -{ -lean_object* x_255; -lean_dec(x_213); -lean_dec(x_212); -lean_dec(x_211); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_255 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_255; -} -} -else -{ -lean_object* x_256; -lean_dec(x_212); -lean_dec(x_211); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_256 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_256; -} -} -else -{ -lean_object* x_257; -lean_dec(x_211); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_257 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_257; -} -} -case 5: -{ -lean_object* x_258; -x_258 = lean_ctor_get(x_210, 0); -lean_inc(x_258); -switch (lean_obj_tag(x_258)) { -case 4: -{ -lean_object* x_259; -x_259 = lean_ctor_get(x_258, 0); -lean_inc(x_259); -lean_dec(x_258); -if (lean_obj_tag(x_259) == 1) -{ -lean_object* x_260; -x_260 = lean_ctor_get(x_259, 0); -lean_inc(x_260); -if (lean_obj_tag(x_260) == 1) -{ -lean_object* x_261; -x_261 = lean_ctor_get(x_260, 0); -lean_inc(x_261); -if (lean_obj_tag(x_261) == 1) -{ -lean_object* x_262; -x_262 = lean_ctor_get(x_261, 0); -lean_inc(x_262); -if (lean_obj_tag(x_262) == 0) -{ -lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; uint8_t x_273; -x_263 = lean_ctor_get(x_1, 1); -lean_inc(x_263); -lean_dec(x_1); -x_264 = lean_ctor_get(x_31, 1); -lean_inc(x_264); -lean_dec(x_31); -x_265 = lean_ctor_get(x_60, 1); -lean_inc(x_265); -lean_dec(x_60); -x_266 = lean_ctor_get(x_129, 1); -lean_inc(x_266); -lean_dec(x_129); -x_267 = lean_ctor_get(x_167, 1); -lean_inc(x_267); -lean_dec(x_167); -x_268 = lean_ctor_get(x_210, 1); -lean_inc(x_268); -lean_dec(x_210); -x_269 = lean_ctor_get(x_259, 1); -lean_inc(x_269); -lean_dec(x_259); -x_270 = lean_ctor_get(x_260, 1); -lean_inc(x_270); -lean_dec(x_260); -x_271 = lean_ctor_get(x_261, 1); -lean_inc(x_271); -lean_dec(x_261); -x_272 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_273 = lean_string_dec_eq(x_271, x_272); -lean_dec(x_271); -if (x_273 == 0) -{ -lean_object* x_274; -lean_dec(x_270); -lean_dec(x_269); -lean_dec(x_268); -lean_dec(x_267); -lean_dec(x_266); -lean_dec(x_265); -lean_dec(x_264); -lean_dec(x_263); -x_274 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_274; -} -else -{ -lean_object* x_275; uint8_t x_276; -x_275 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_276 = lean_string_dec_eq(x_270, x_275); -lean_dec(x_270); -if (x_276 == 0) -{ -lean_object* x_277; -lean_dec(x_269); -lean_dec(x_268); -lean_dec(x_267); -lean_dec(x_266); -lean_dec(x_265); -lean_dec(x_264); -lean_dec(x_263); -x_277 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_277; -} -else -{ -lean_object* x_278; uint8_t x_279; -x_278 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__10; -x_279 = lean_string_dec_eq(x_269, x_278); -lean_dec(x_269); -if (x_279 == 0) -{ -lean_object* x_280; -lean_dec(x_268); -lean_dec(x_267); -lean_dec(x_266); -lean_dec(x_265); -lean_dec(x_264); -lean_dec(x_263); -x_280 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_280; -} -else -{ -if (lean_obj_tag(x_268) == 9) -{ -lean_object* x_281; -x_281 = lean_ctor_get(x_268, 0); -lean_inc(x_281); -lean_dec(x_268); -if (lean_obj_tag(x_281) == 0) -{ -lean_object* x_282; -lean_dec(x_281); -lean_dec(x_267); -lean_dec(x_266); -lean_dec(x_265); -lean_dec(x_264); -lean_dec(x_263); -x_282 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_282; -} -else -{ -if (lean_obj_tag(x_267) == 9) -{ -lean_object* x_283; -x_283 = lean_ctor_get(x_267, 0); -lean_inc(x_283); -lean_dec(x_267); -if (lean_obj_tag(x_283) == 0) -{ -lean_object* x_284; -lean_dec(x_283); -lean_dec(x_281); -lean_dec(x_266); -lean_dec(x_265); -lean_dec(x_264); -lean_dec(x_263); -x_284 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_284; -} -else -{ -if (lean_obj_tag(x_266) == 9) -{ -lean_object* x_285; -x_285 = lean_ctor_get(x_266, 0); -lean_inc(x_285); -lean_dec(x_266); -if (lean_obj_tag(x_285) == 0) -{ -lean_object* x_286; -lean_dec(x_285); -lean_dec(x_283); -lean_dec(x_281); -lean_dec(x_265); -lean_dec(x_264); -lean_dec(x_263); -x_286 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_286; -} -else -{ -if (lean_obj_tag(x_265) == 9) -{ -lean_object* x_287; -x_287 = lean_ctor_get(x_265, 0); -lean_inc(x_287); -lean_dec(x_265); -if (lean_obj_tag(x_287) == 0) -{ -lean_object* x_288; -lean_dec(x_287); -lean_dec(x_285); -lean_dec(x_283); -lean_dec(x_281); -lean_dec(x_264); -lean_dec(x_263); -x_288 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_288; -} -else -{ -if (lean_obj_tag(x_264) == 9) -{ -lean_object* x_289; -x_289 = lean_ctor_get(x_264, 0); -lean_inc(x_289); -lean_dec(x_264); -if (lean_obj_tag(x_289) == 0) -{ -lean_object* x_290; -lean_dec(x_289); -lean_dec(x_287); -lean_dec(x_285); -lean_dec(x_283); -lean_dec(x_281); -lean_dec(x_263); -x_290 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_290; -} -else -{ -if (lean_obj_tag(x_263) == 9) -{ -lean_object* x_291; -x_291 = lean_ctor_get(x_263, 0); -lean_inc(x_291); -lean_dec(x_263); -if (lean_obj_tag(x_291) == 0) -{ -lean_object* x_292; -lean_dec(x_291); -lean_dec(x_289); -lean_dec(x_287); -lean_dec(x_285); -lean_dec(x_283); -lean_dec(x_281); -x_292 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_292; -} -else -{ -lean_object* x_293; lean_object* x_294; lean_object* x_295; lean_object* x_296; lean_object* x_297; lean_object* x_298; lean_object* x_299; lean_object* x_300; -x_293 = lean_ctor_get(x_281, 0); -lean_inc(x_293); -lean_dec(x_281); -x_294 = lean_ctor_get(x_283, 0); -lean_inc(x_294); -lean_dec(x_283); -x_295 = lean_ctor_get(x_285, 0); -lean_inc(x_295); -lean_dec(x_285); -x_296 = lean_ctor_get(x_287, 0); -lean_inc(x_296); -lean_dec(x_287); -x_297 = lean_ctor_get(x_289, 0); -lean_inc(x_297); -lean_dec(x_289); -x_298 = lean_ctor_get(x_291, 0); -lean_inc(x_298); -lean_dec(x_291); -x_299 = l_Lean_Name_mkStr6(x_293, x_294, x_295, x_296, x_297, x_298); -x_300 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_300, 0, x_299); -lean_ctor_set(x_300, 1, x_8); -return x_300; -} -} -else -{ -lean_object* x_301; -lean_dec(x_289); -lean_dec(x_287); -lean_dec(x_285); -lean_dec(x_283); -lean_dec(x_281); -lean_dec(x_263); -x_301 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_301; -} -} -} -else -{ -lean_object* x_302; -lean_dec(x_287); -lean_dec(x_285); -lean_dec(x_283); -lean_dec(x_281); -lean_dec(x_264); -lean_dec(x_263); -x_302 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_302; -} -} -} -else -{ -lean_object* x_303; -lean_dec(x_285); -lean_dec(x_283); -lean_dec(x_281); -lean_dec(x_265); -lean_dec(x_264); -lean_dec(x_263); -x_303 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_303; -} -} -} -else -{ -lean_object* x_304; -lean_dec(x_283); -lean_dec(x_281); -lean_dec(x_266); -lean_dec(x_265); -lean_dec(x_264); -lean_dec(x_263); -x_304 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_304; -} -} -} -else -{ -lean_object* x_305; -lean_dec(x_281); -lean_dec(x_267); -lean_dec(x_266); -lean_dec(x_265); -lean_dec(x_264); -lean_dec(x_263); -x_305 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_305; -} -} -} -else -{ -lean_object* x_306; -lean_dec(x_268); -lean_dec(x_267); -lean_dec(x_266); -lean_dec(x_265); -lean_dec(x_264); -lean_dec(x_263); -x_306 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_306; -} -} -} -} -} -else -{ -lean_object* x_307; -lean_dec(x_262); -lean_dec(x_261); -lean_dec(x_260); -lean_dec(x_259); -lean_dec(x_210); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_307 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_307; -} -} -else -{ -lean_object* x_308; -lean_dec(x_261); -lean_dec(x_260); -lean_dec(x_259); -lean_dec(x_210); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_308 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_308; -} -} -else -{ -lean_object* x_309; -lean_dec(x_260); -lean_dec(x_259); -lean_dec(x_210); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_309 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_309; -} -} -else -{ -lean_object* x_310; -lean_dec(x_259); -lean_dec(x_210); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_310 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_310; -} -} -case 5: -{ -lean_object* x_311; -x_311 = lean_ctor_get(x_258, 0); -lean_inc(x_311); -switch (lean_obj_tag(x_311)) { -case 4: -{ -lean_object* x_312; -x_312 = lean_ctor_get(x_311, 0); -lean_inc(x_312); -lean_dec(x_311); -if (lean_obj_tag(x_312) == 1) -{ -lean_object* x_313; -x_313 = lean_ctor_get(x_312, 0); -lean_inc(x_313); -if (lean_obj_tag(x_313) == 1) -{ -lean_object* x_314; -x_314 = lean_ctor_get(x_313, 0); -lean_inc(x_314); -if (lean_obj_tag(x_314) == 1) -{ -lean_object* x_315; -x_315 = lean_ctor_get(x_314, 0); -lean_inc(x_315); -if (lean_obj_tag(x_315) == 0) -{ -lean_object* x_316; lean_object* x_317; lean_object* x_318; lean_object* x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; lean_object* x_324; lean_object* x_325; lean_object* x_326; uint8_t x_327; -x_316 = lean_ctor_get(x_1, 1); -lean_inc(x_316); -lean_dec(x_1); -x_317 = lean_ctor_get(x_31, 1); -lean_inc(x_317); -lean_dec(x_31); -x_318 = lean_ctor_get(x_60, 1); -lean_inc(x_318); -lean_dec(x_60); -x_319 = lean_ctor_get(x_129, 1); -lean_inc(x_319); -lean_dec(x_129); -x_320 = lean_ctor_get(x_167, 1); -lean_inc(x_320); -lean_dec(x_167); -x_321 = lean_ctor_get(x_210, 1); -lean_inc(x_321); -lean_dec(x_210); -x_322 = lean_ctor_get(x_258, 1); -lean_inc(x_322); -lean_dec(x_258); -x_323 = lean_ctor_get(x_312, 1); -lean_inc(x_323); -lean_dec(x_312); -x_324 = lean_ctor_get(x_313, 1); -lean_inc(x_324); -lean_dec(x_313); -x_325 = lean_ctor_get(x_314, 1); -lean_inc(x_325); -lean_dec(x_314); -x_326 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_327 = lean_string_dec_eq(x_325, x_326); -lean_dec(x_325); -if (x_327 == 0) -{ -lean_object* x_328; -lean_dec(x_324); -lean_dec(x_323); -lean_dec(x_322); -lean_dec(x_321); -lean_dec(x_320); -lean_dec(x_319); -lean_dec(x_318); -lean_dec(x_317); -lean_dec(x_316); -x_328 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_328; -} -else -{ -lean_object* x_329; uint8_t x_330; -x_329 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_330 = lean_string_dec_eq(x_324, x_329); -lean_dec(x_324); -if (x_330 == 0) -{ -lean_object* x_331; -lean_dec(x_323); -lean_dec(x_322); -lean_dec(x_321); -lean_dec(x_320); -lean_dec(x_319); -lean_dec(x_318); -lean_dec(x_317); -lean_dec(x_316); -x_331 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_331; -} -else -{ -lean_object* x_332; uint8_t x_333; -x_332 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__11; -x_333 = lean_string_dec_eq(x_323, x_332); -lean_dec(x_323); -if (x_333 == 0) -{ -lean_object* x_334; -lean_dec(x_322); -lean_dec(x_321); -lean_dec(x_320); -lean_dec(x_319); -lean_dec(x_318); -lean_dec(x_317); -lean_dec(x_316); -x_334 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_334; -} -else -{ -if (lean_obj_tag(x_322) == 9) -{ -lean_object* x_335; -x_335 = lean_ctor_get(x_322, 0); -lean_inc(x_335); -lean_dec(x_322); -if (lean_obj_tag(x_335) == 0) -{ -lean_object* x_336; -lean_dec(x_335); -lean_dec(x_321); -lean_dec(x_320); -lean_dec(x_319); -lean_dec(x_318); -lean_dec(x_317); -lean_dec(x_316); -x_336 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_336; -} -else -{ -if (lean_obj_tag(x_321) == 9) -{ -lean_object* x_337; -x_337 = lean_ctor_get(x_321, 0); -lean_inc(x_337); -lean_dec(x_321); -if (lean_obj_tag(x_337) == 0) -{ -lean_object* x_338; -lean_dec(x_337); -lean_dec(x_335); -lean_dec(x_320); -lean_dec(x_319); -lean_dec(x_318); -lean_dec(x_317); -lean_dec(x_316); -x_338 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_338; -} -else -{ -if (lean_obj_tag(x_320) == 9) -{ -lean_object* x_339; -x_339 = lean_ctor_get(x_320, 0); -lean_inc(x_339); -lean_dec(x_320); -if (lean_obj_tag(x_339) == 0) -{ -lean_object* x_340; -lean_dec(x_339); -lean_dec(x_337); -lean_dec(x_335); -lean_dec(x_319); -lean_dec(x_318); -lean_dec(x_317); -lean_dec(x_316); -x_340 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_340; -} -else -{ -if (lean_obj_tag(x_319) == 9) -{ -lean_object* x_341; -x_341 = lean_ctor_get(x_319, 0); -lean_inc(x_341); -lean_dec(x_319); -if (lean_obj_tag(x_341) == 0) -{ -lean_object* x_342; -lean_dec(x_341); -lean_dec(x_339); -lean_dec(x_337); -lean_dec(x_335); -lean_dec(x_318); -lean_dec(x_317); -lean_dec(x_316); -x_342 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_342; -} -else -{ -if (lean_obj_tag(x_318) == 9) -{ -lean_object* x_343; -x_343 = lean_ctor_get(x_318, 0); -lean_inc(x_343); -lean_dec(x_318); -if (lean_obj_tag(x_343) == 0) -{ -lean_object* x_344; -lean_dec(x_343); -lean_dec(x_341); -lean_dec(x_339); -lean_dec(x_337); -lean_dec(x_335); -lean_dec(x_317); -lean_dec(x_316); -x_344 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_344; -} -else -{ -if (lean_obj_tag(x_317) == 9) -{ -lean_object* x_345; -x_345 = lean_ctor_get(x_317, 0); -lean_inc(x_345); -lean_dec(x_317); -if (lean_obj_tag(x_345) == 0) -{ -lean_object* x_346; -lean_dec(x_345); -lean_dec(x_343); -lean_dec(x_341); -lean_dec(x_339); -lean_dec(x_337); -lean_dec(x_335); -lean_dec(x_316); -x_346 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_346; -} -else -{ -if (lean_obj_tag(x_316) == 9) -{ -lean_object* x_347; -x_347 = lean_ctor_get(x_316, 0); -lean_inc(x_347); -lean_dec(x_316); -if (lean_obj_tag(x_347) == 0) -{ -lean_object* x_348; -lean_dec(x_347); -lean_dec(x_345); -lean_dec(x_343); -lean_dec(x_341); -lean_dec(x_339); -lean_dec(x_337); -lean_dec(x_335); -x_348 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_348; -} -else -{ -lean_object* x_349; lean_object* x_350; lean_object* x_351; lean_object* x_352; lean_object* x_353; lean_object* x_354; lean_object* x_355; lean_object* x_356; lean_object* x_357; -x_349 = lean_ctor_get(x_335, 0); -lean_inc(x_349); -lean_dec(x_335); -x_350 = lean_ctor_get(x_337, 0); -lean_inc(x_350); -lean_dec(x_337); -x_351 = lean_ctor_get(x_339, 0); -lean_inc(x_351); -lean_dec(x_339); -x_352 = lean_ctor_get(x_341, 0); -lean_inc(x_352); -lean_dec(x_341); -x_353 = lean_ctor_get(x_343, 0); -lean_inc(x_353); -lean_dec(x_343); -x_354 = lean_ctor_get(x_345, 0); -lean_inc(x_354); -lean_dec(x_345); -x_355 = lean_ctor_get(x_347, 0); -lean_inc(x_355); -lean_dec(x_347); -x_356 = l_Lean_Name_mkStr7(x_349, x_350, x_351, x_352, x_353, x_354, x_355); -x_357 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_357, 0, x_356); -lean_ctor_set(x_357, 1, x_8); -return x_357; -} -} -else -{ -lean_object* x_358; -lean_dec(x_345); -lean_dec(x_343); -lean_dec(x_341); -lean_dec(x_339); -lean_dec(x_337); -lean_dec(x_335); -lean_dec(x_316); -x_358 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_358; -} -} -} -else -{ -lean_object* x_359; -lean_dec(x_343); -lean_dec(x_341); -lean_dec(x_339); -lean_dec(x_337); -lean_dec(x_335); -lean_dec(x_317); -lean_dec(x_316); -x_359 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_359; -} -} -} -else -{ -lean_object* x_360; -lean_dec(x_341); -lean_dec(x_339); -lean_dec(x_337); -lean_dec(x_335); -lean_dec(x_318); -lean_dec(x_317); -lean_dec(x_316); -x_360 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_360; -} -} -} -else -{ -lean_object* x_361; -lean_dec(x_339); -lean_dec(x_337); -lean_dec(x_335); -lean_dec(x_319); -lean_dec(x_318); -lean_dec(x_317); -lean_dec(x_316); -x_361 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_361; -} -} -} -else -{ -lean_object* x_362; -lean_dec(x_337); -lean_dec(x_335); -lean_dec(x_320); -lean_dec(x_319); -lean_dec(x_318); -lean_dec(x_317); -lean_dec(x_316); -x_362 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_362; -} -} -} -else -{ -lean_object* x_363; -lean_dec(x_335); -lean_dec(x_321); -lean_dec(x_320); -lean_dec(x_319); -lean_dec(x_318); -lean_dec(x_317); -lean_dec(x_316); -x_363 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_363; -} -} -} -else -{ -lean_object* x_364; -lean_dec(x_322); -lean_dec(x_321); -lean_dec(x_320); -lean_dec(x_319); -lean_dec(x_318); -lean_dec(x_317); -lean_dec(x_316); -x_364 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_364; -} -} -} -} -} -else -{ -lean_object* x_365; -lean_dec(x_315); -lean_dec(x_314); -lean_dec(x_313); -lean_dec(x_312); -lean_dec(x_258); -lean_dec(x_210); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_365 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_365; -} -} -else -{ -lean_object* x_366; -lean_dec(x_314); -lean_dec(x_313); -lean_dec(x_312); -lean_dec(x_258); -lean_dec(x_210); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_366 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_366; -} -} -else -{ -lean_object* x_367; -lean_dec(x_313); -lean_dec(x_312); -lean_dec(x_258); -lean_dec(x_210); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_367 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_367; -} -} -else -{ -lean_object* x_368; -lean_dec(x_312); -lean_dec(x_258); -lean_dec(x_210); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_368 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_368; -} -} -case 5: -{ -lean_object* x_369; -x_369 = lean_ctor_get(x_311, 0); -lean_inc(x_369); -if (lean_obj_tag(x_369) == 4) -{ -lean_object* x_370; -x_370 = lean_ctor_get(x_369, 0); -lean_inc(x_370); -lean_dec(x_369); -if (lean_obj_tag(x_370) == 1) -{ -lean_object* x_371; -x_371 = lean_ctor_get(x_370, 0); -lean_inc(x_371); -if (lean_obj_tag(x_371) == 1) -{ -lean_object* x_372; -x_372 = lean_ctor_get(x_371, 0); -lean_inc(x_372); -if (lean_obj_tag(x_372) == 1) -{ -lean_object* x_373; -x_373 = lean_ctor_get(x_372, 0); -lean_inc(x_373); -if (lean_obj_tag(x_373) == 0) -{ -lean_object* x_374; lean_object* x_375; lean_object* x_376; lean_object* x_377; lean_object* x_378; lean_object* x_379; lean_object* x_380; lean_object* x_381; lean_object* x_382; lean_object* x_383; lean_object* x_384; lean_object* x_385; uint8_t x_386; -x_374 = lean_ctor_get(x_1, 1); -lean_inc(x_374); -lean_dec(x_1); -x_375 = lean_ctor_get(x_31, 1); -lean_inc(x_375); -lean_dec(x_31); -x_376 = lean_ctor_get(x_60, 1); -lean_inc(x_376); -lean_dec(x_60); -x_377 = lean_ctor_get(x_129, 1); -lean_inc(x_377); -lean_dec(x_129); -x_378 = lean_ctor_get(x_167, 1); -lean_inc(x_378); -lean_dec(x_167); -x_379 = lean_ctor_get(x_210, 1); -lean_inc(x_379); -lean_dec(x_210); -x_380 = lean_ctor_get(x_258, 1); -lean_inc(x_380); -lean_dec(x_258); -x_381 = lean_ctor_get(x_311, 1); -lean_inc(x_381); -lean_dec(x_311); -x_382 = lean_ctor_get(x_370, 1); -lean_inc(x_382); -lean_dec(x_370); -x_383 = lean_ctor_get(x_371, 1); -lean_inc(x_383); -lean_dec(x_371); -x_384 = lean_ctor_get(x_372, 1); -lean_inc(x_384); -lean_dec(x_372); -x_385 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_386 = lean_string_dec_eq(x_384, x_385); -lean_dec(x_384); -if (x_386 == 0) -{ -lean_object* x_387; -lean_dec(x_383); -lean_dec(x_382); -lean_dec(x_381); -lean_dec(x_380); -lean_dec(x_379); -lean_dec(x_378); -lean_dec(x_377); -lean_dec(x_376); -lean_dec(x_375); -lean_dec(x_374); -x_387 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_387; -} -else -{ -lean_object* x_388; uint8_t x_389; -x_388 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_389 = lean_string_dec_eq(x_383, x_388); -lean_dec(x_383); -if (x_389 == 0) -{ -lean_object* x_390; -lean_dec(x_382); -lean_dec(x_381); -lean_dec(x_380); -lean_dec(x_379); -lean_dec(x_378); -lean_dec(x_377); -lean_dec(x_376); -lean_dec(x_375); -lean_dec(x_374); -x_390 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_390; -} -else -{ -lean_object* x_391; uint8_t x_392; -x_391 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__12; -x_392 = lean_string_dec_eq(x_382, x_391); -lean_dec(x_382); -if (x_392 == 0) -{ -lean_object* x_393; -lean_dec(x_381); -lean_dec(x_380); -lean_dec(x_379); -lean_dec(x_378); -lean_dec(x_377); -lean_dec(x_376); -lean_dec(x_375); -lean_dec(x_374); -x_393 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_393; -} -else -{ -if (lean_obj_tag(x_381) == 9) -{ -lean_object* x_394; -x_394 = lean_ctor_get(x_381, 0); -lean_inc(x_394); -lean_dec(x_381); -if (lean_obj_tag(x_394) == 0) -{ -lean_object* x_395; -lean_dec(x_394); -lean_dec(x_380); -lean_dec(x_379); -lean_dec(x_378); -lean_dec(x_377); -lean_dec(x_376); -lean_dec(x_375); -lean_dec(x_374); -x_395 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_395; -} -else -{ -if (lean_obj_tag(x_380) == 9) -{ -lean_object* x_396; -x_396 = lean_ctor_get(x_380, 0); -lean_inc(x_396); -lean_dec(x_380); -if (lean_obj_tag(x_396) == 0) -{ -lean_object* x_397; -lean_dec(x_396); -lean_dec(x_394); -lean_dec(x_379); -lean_dec(x_378); -lean_dec(x_377); -lean_dec(x_376); -lean_dec(x_375); -lean_dec(x_374); -x_397 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_397; -} -else -{ -if (lean_obj_tag(x_379) == 9) -{ -lean_object* x_398; -x_398 = lean_ctor_get(x_379, 0); -lean_inc(x_398); -lean_dec(x_379); -if (lean_obj_tag(x_398) == 0) -{ -lean_object* x_399; -lean_dec(x_398); -lean_dec(x_396); -lean_dec(x_394); -lean_dec(x_378); -lean_dec(x_377); -lean_dec(x_376); -lean_dec(x_375); -lean_dec(x_374); -x_399 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_399; -} -else -{ -if (lean_obj_tag(x_378) == 9) -{ -lean_object* x_400; -x_400 = lean_ctor_get(x_378, 0); -lean_inc(x_400); -lean_dec(x_378); -if (lean_obj_tag(x_400) == 0) -{ -lean_object* x_401; -lean_dec(x_400); -lean_dec(x_398); -lean_dec(x_396); -lean_dec(x_394); -lean_dec(x_377); -lean_dec(x_376); -lean_dec(x_375); -lean_dec(x_374); -x_401 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_401; -} -else -{ -if (lean_obj_tag(x_377) == 9) -{ -lean_object* x_402; -x_402 = lean_ctor_get(x_377, 0); -lean_inc(x_402); -lean_dec(x_377); -if (lean_obj_tag(x_402) == 0) -{ -lean_object* x_403; -lean_dec(x_402); -lean_dec(x_400); -lean_dec(x_398); -lean_dec(x_396); -lean_dec(x_394); -lean_dec(x_376); -lean_dec(x_375); -lean_dec(x_374); -x_403 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_403; -} -else -{ -if (lean_obj_tag(x_376) == 9) -{ -lean_object* x_404; -x_404 = lean_ctor_get(x_376, 0); -lean_inc(x_404); -lean_dec(x_376); -if (lean_obj_tag(x_404) == 0) -{ -lean_object* x_405; -lean_dec(x_404); -lean_dec(x_402); -lean_dec(x_400); -lean_dec(x_398); -lean_dec(x_396); -lean_dec(x_394); -lean_dec(x_375); -lean_dec(x_374); -x_405 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_405; -} -else -{ -if (lean_obj_tag(x_375) == 9) -{ -lean_object* x_406; -x_406 = lean_ctor_get(x_375, 0); -lean_inc(x_406); -lean_dec(x_375); -if (lean_obj_tag(x_406) == 0) -{ -lean_object* x_407; -lean_dec(x_406); -lean_dec(x_404); -lean_dec(x_402); -lean_dec(x_400); -lean_dec(x_398); -lean_dec(x_396); -lean_dec(x_394); -lean_dec(x_374); -x_407 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_407; -} -else -{ -if (lean_obj_tag(x_374) == 9) -{ -lean_object* x_408; -x_408 = lean_ctor_get(x_374, 0); -lean_inc(x_408); -lean_dec(x_374); -if (lean_obj_tag(x_408) == 0) -{ -lean_object* x_409; -lean_dec(x_408); -lean_dec(x_406); -lean_dec(x_404); -lean_dec(x_402); -lean_dec(x_400); -lean_dec(x_398); -lean_dec(x_396); -lean_dec(x_394); -x_409 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_409; -} -else -{ -lean_object* x_410; lean_object* x_411; lean_object* x_412; lean_object* x_413; lean_object* x_414; lean_object* x_415; lean_object* x_416; lean_object* x_417; lean_object* x_418; lean_object* x_419; -x_410 = lean_ctor_get(x_394, 0); -lean_inc(x_410); -lean_dec(x_394); -x_411 = lean_ctor_get(x_396, 0); -lean_inc(x_411); -lean_dec(x_396); -x_412 = lean_ctor_get(x_398, 0); -lean_inc(x_412); -lean_dec(x_398); -x_413 = lean_ctor_get(x_400, 0); -lean_inc(x_413); -lean_dec(x_400); -x_414 = lean_ctor_get(x_402, 0); -lean_inc(x_414); -lean_dec(x_402); -x_415 = lean_ctor_get(x_404, 0); -lean_inc(x_415); -lean_dec(x_404); -x_416 = lean_ctor_get(x_406, 0); -lean_inc(x_416); -lean_dec(x_406); -x_417 = lean_ctor_get(x_408, 0); -lean_inc(x_417); -lean_dec(x_408); -x_418 = l_Lean_Name_mkStr8(x_410, x_411, x_412, x_413, x_414, x_415, x_416, x_417); -x_419 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_419, 0, x_418); -lean_ctor_set(x_419, 1, x_8); -return x_419; -} -} -else -{ -lean_object* x_420; -lean_dec(x_406); -lean_dec(x_404); -lean_dec(x_402); -lean_dec(x_400); -lean_dec(x_398); -lean_dec(x_396); -lean_dec(x_394); -lean_dec(x_374); -x_420 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_420; -} -} -} -else -{ -lean_object* x_421; -lean_dec(x_404); -lean_dec(x_402); -lean_dec(x_400); -lean_dec(x_398); -lean_dec(x_396); -lean_dec(x_394); -lean_dec(x_375); -lean_dec(x_374); -x_421 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_421; -} -} -} -else -{ -lean_object* x_422; -lean_dec(x_402); -lean_dec(x_400); -lean_dec(x_398); -lean_dec(x_396); -lean_dec(x_394); -lean_dec(x_376); -lean_dec(x_375); -lean_dec(x_374); -x_422 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_422; -} -} -} -else -{ -lean_object* x_423; -lean_dec(x_400); -lean_dec(x_398); -lean_dec(x_396); -lean_dec(x_394); -lean_dec(x_377); -lean_dec(x_376); -lean_dec(x_375); -lean_dec(x_374); -x_423 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_423; -} -} -} -else -{ -lean_object* x_424; -lean_dec(x_398); -lean_dec(x_396); -lean_dec(x_394); -lean_dec(x_378); -lean_dec(x_377); -lean_dec(x_376); -lean_dec(x_375); -lean_dec(x_374); -x_424 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_424; -} -} -} -else -{ -lean_object* x_425; -lean_dec(x_396); -lean_dec(x_394); -lean_dec(x_379); -lean_dec(x_378); -lean_dec(x_377); -lean_dec(x_376); -lean_dec(x_375); -lean_dec(x_374); -x_425 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_425; -} -} -} -else -{ -lean_object* x_426; -lean_dec(x_394); -lean_dec(x_380); -lean_dec(x_379); -lean_dec(x_378); -lean_dec(x_377); -lean_dec(x_376); -lean_dec(x_375); -lean_dec(x_374); -x_426 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_426; -} -} -} -else -{ -lean_object* x_427; -lean_dec(x_381); -lean_dec(x_380); -lean_dec(x_379); -lean_dec(x_378); -lean_dec(x_377); -lean_dec(x_376); -lean_dec(x_375); -lean_dec(x_374); -x_427 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_427; -} -} -} -} -} -else -{ -lean_object* x_428; -lean_dec(x_373); -lean_dec(x_372); -lean_dec(x_371); -lean_dec(x_370); -lean_dec(x_311); -lean_dec(x_258); -lean_dec(x_210); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_428 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_428; -} -} -else -{ -lean_object* x_429; -lean_dec(x_372); -lean_dec(x_371); -lean_dec(x_370); -lean_dec(x_311); -lean_dec(x_258); -lean_dec(x_210); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_429 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_429; -} -} -else -{ -lean_object* x_430; -lean_dec(x_371); -lean_dec(x_370); -lean_dec(x_311); -lean_dec(x_258); -lean_dec(x_210); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_430 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_430; -} -} -else -{ -lean_object* x_431; -lean_dec(x_370); -lean_dec(x_311); -lean_dec(x_258); -lean_dec(x_210); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_431 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_431; -} -} -else -{ -lean_object* x_432; -lean_dec(x_369); -lean_dec(x_311); -lean_dec(x_258); -lean_dec(x_210); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_432 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_432; -} -} -default: -{ -lean_object* x_433; -lean_dec(x_311); -lean_dec(x_258); -lean_dec(x_210); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_433 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_433; -} -} -} -default: -{ -lean_object* x_434; -lean_dec(x_258); -lean_dec(x_210); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_434 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_434; -} -} -} -default: -{ -lean_object* x_435; -lean_dec(x_210); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_435 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_435; -} -} -} -default: -{ -lean_object* x_436; -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_436 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_436; -} -} -} -default: -{ -lean_object* x_437; -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_437 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_437; -} -} -} -default: -{ -lean_object* x_438; -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_438 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_438; -} -} -} -default: -{ -lean_object* x_439; -lean_dec(x_31); -lean_dec(x_1); -x_439 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_439; -} -} -} -default: -{ -lean_object* x_440; -lean_dec(x_1); -x_440 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_440; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_reifyName___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; -x_9 = l_Lean_PrettyPrinter_Delaborator_reifyName(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_9; -} -} -LEAN_EXPORT uint8_t l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__1(lean_object* x_1) { -_start: -{ -uint8_t x_2; -x_2 = 0; -return x_2; -} -} -static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("quotedName", 10, 10); -return x_1; -} -} -static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_2 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__3; -x_3 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__4; -x_4 = l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__1; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; -} -} -static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__1___boxed), 1, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("`", 1, 1); -return x_1; -} -} -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; -x_9 = l_Lean_PrettyPrinter_Delaborator_reifyName(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_9) == 0) -{ -uint8_t x_10; -x_10 = !lean_is_exclusive(x_9); -if (x_10 == 0) -{ -lean_object* x_11; uint8_t x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_11 = lean_ctor_get(x_9, 0); -x_12 = 1; -x_13 = l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__3; -x_14 = l_Lean_Name_toString(x_11, x_12, x_13); -x_15 = l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__4; -x_16 = lean_string_append(x_15, x_14); -lean_dec(x_14); -x_17 = l_Lean_PrettyPrinter_Delaborator_delabOfScientific___lambda__1___closed__2; -x_18 = lean_string_append(x_16, x_17); -x_19 = lean_box(2); -x_20 = l_Lean_Syntax_mkNameLit(x_18, x_19); -x_21 = lean_box(0); -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_array_mk(x_22); -x_24 = l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__2; -x_25 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_25, 0, x_19); -lean_ctor_set(x_25, 1, x_24); -lean_ctor_set(x_25, 2, x_23); -lean_ctor_set(x_9, 0, x_25); -return x_9; -} -else -{ -lean_object* x_26; lean_object* x_27; uint8_t x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_26 = lean_ctor_get(x_9, 0); -x_27 = lean_ctor_get(x_9, 1); -lean_inc(x_27); -lean_inc(x_26); -lean_dec(x_9); -x_28 = 1; -x_29 = l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__3; -x_30 = l_Lean_Name_toString(x_26, x_28, x_29); -x_31 = l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__4; -x_32 = lean_string_append(x_31, x_30); -lean_dec(x_30); -x_33 = l_Lean_PrettyPrinter_Delaborator_delabOfScientific___lambda__1___closed__2; -x_34 = lean_string_append(x_32, x_33); -x_35 = lean_box(2); -x_36 = l_Lean_Syntax_mkNameLit(x_34, x_35); -x_37 = lean_box(0); -x_38 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -x_39 = lean_array_mk(x_38); -x_40 = l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__2; -x_41 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_41, 0, x_35); -lean_ctor_set(x_41, 1, x_40); -lean_ctor_set(x_41, 2, x_39); -x_42 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_42, 0, x_41); -lean_ctor_set(x_42, 1, x_27); -return x_42; -} -} -else -{ -uint8_t x_43; -x_43 = !lean_is_exclusive(x_9); -if (x_43 == 0) -{ -return x_9; -} -else -{ -lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_44 = lean_ctor_get(x_9, 0); -x_45 = lean_ctor_get(x_9, 1); -lean_inc(x_45); -lean_inc(x_44); -lean_dec(x_9); -x_46 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_46, 0, x_44); -lean_ctor_set(x_46, 1, x_45); -return x_46; -} -} -} -} -static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___closed__1() { -_start: +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__9___closed__1() { +_start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___boxed), 8, 0); +x_1 = lean_mk_string_unchecked("mkStr8", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_PrettyPrinter_Delaborator_delabAppExplicitCore___closed__1; -x_2 = l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___closed__1; -x_3 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_PrettyPrinter_Delaborator_delabMVarAux___spec__1___rarg), 9, 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_Delaborator_delabNameMkStr(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; -x_8 = l_Lean_PrettyPrinter_Delaborator_delabAppImplicitCore___lambda__11___closed__2; -x_9 = l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___closed__2; -x_10 = l_Lean_PrettyPrinter_Delaborator_whenPPOption(x_8, x_9, x_1, x_2, x_3, x_4, x_5, x_6, x_7); -return x_10; -} -} -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__1___boxed(lean_object* x_1) { -_start: -{ -uint8_t x_2; lean_object* x_3; -x_2 = l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__1(x_1); -lean_dec(x_1); -x_3 = lean_box(x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; -x_9 = l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_9; -} -} -static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__9___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabApp__1___closed__1; x_2 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_3 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_4 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__4; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; -} -} -static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__2() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("delabNameMkStr", 14, 14); -return x_1; -} -} -static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_2 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabFVar__1___closed__3; -x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabFVar__1___closed__4; -x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__2; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; -} -} -static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Delaborator_delabNameMkStr), 7, 0); -return x_1; -} -} -LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_2 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabFVar__1___closed__7; x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__1; -x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__3; -x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__4; -x_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_PrettyPrinter_Delaborator_delabNameMkStr__2___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___regBuiltin_Lean_PrettyPrinter_Delaborator_delabApp__1___closed__1; -x_2 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_3 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_4 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__3; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; -} -} -LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__2(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_2 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabFVar__1___closed__7; -x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__2___closed__1; -x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__3; -x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__4; -x_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_PrettyPrinter_Delaborator_delabNameMkStr__3___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___regBuiltin_Lean_PrettyPrinter_Delaborator_delabApp__1___closed__1; -x_2 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_3 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_4 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__6; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; -} -} -LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__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; -x_2 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabFVar__1___closed__7; -x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__3___closed__1; -x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__3; -x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__4; -x_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_PrettyPrinter_Delaborator_delabNameMkStr__4___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___regBuiltin_Lean_PrettyPrinter_Delaborator_delabApp__1___closed__1; -x_2 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_3 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_4 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__7; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; -} -} -LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__4(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_2 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabFVar__1___closed__7; -x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__4___closed__1; -x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__3; -x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__4; -x_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_PrettyPrinter_Delaborator_delabNameMkStr__5___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___regBuiltin_Lean_PrettyPrinter_Delaborator_delabApp__1___closed__1; -x_2 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_3 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_4 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__8; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; -} -} -LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__5(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_2 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabFVar__1___closed__7; -x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__5___closed__1; -x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__3; -x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__4; -x_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_PrettyPrinter_Delaborator_delabNameMkStr__6___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___regBuiltin_Lean_PrettyPrinter_Delaborator_delabApp__1___closed__1; -x_2 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_3 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_4 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__9; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; -} -} -LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__6(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_2 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabFVar__1___closed__7; -x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__6___closed__1; -x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__3; -x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__4; -x_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_PrettyPrinter_Delaborator_delabNameMkStr__7___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___regBuiltin_Lean_PrettyPrinter_Delaborator_delabApp__1___closed__1; -x_2 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_3 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_4 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__10; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; -} -} -LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__7(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_2 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabFVar__1___closed__7; -x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__7___closed__1; -x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__3; -x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__4; -x_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_PrettyPrinter_Delaborator_delabNameMkStr__8___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___regBuiltin_Lean_PrettyPrinter_Delaborator_delabApp__1___closed__1; -x_2 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_3 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_4 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__11; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; -} -} -LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__8(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_2 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabFVar__1___closed__7; -x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__8___closed__1; -x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__3; -x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__4; -x_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_PrettyPrinter_Delaborator_delabNameMkStr__9___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___regBuiltin_Lean_PrettyPrinter_Delaborator_delabApp__1___closed__1; -x_2 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_3 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_4 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__12; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__9___closed__1; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } @@ -48707,9 +45742,9 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabName { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_2 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabFVar__1___closed__7; -x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__9___closed__1; -x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__3; -x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__4; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__9___closed__2; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__5; +x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__6; x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); return x_6; } @@ -48725,16 +45760,24 @@ return x_8; static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__1() { _start: { +lean_object* x_1; +x_1 = lean_mk_string_unchecked("num", 3, 3); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__2() { +_start: +{ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabApp__1___closed__1; x_2 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_3 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_4 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__5; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__1; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__1; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__2() { +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__3() { _start: { lean_object* x_1; @@ -48742,19 +45785,19 @@ x_1 = lean_mk_string_unchecked("delabNameMkNum", 14, 14); return x_1; } } -static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__3() { +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; x_2 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabFVar__1___closed__3; x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabFVar__1___closed__4; -x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__2; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__3; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__4() { +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__5() { _start: { lean_object* x_1; @@ -48767,9 +45810,9 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabName { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_2 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabFVar__1___closed__7; -x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__1; -x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__3; -x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__4; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__2; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__4; +x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__5; x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); return x_6; } @@ -51792,7 +48835,7 @@ static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_delabConstWithSignatu lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_PrettyPrinter_Delaborator_delabFVar___closed__1; x_2 = l_Lean_PrettyPrinter_Delaborator_delabConstWithSignature_delabParamsAux___closed__1; -x_3 = lean_unsigned_to_nat(1307u); +x_3 = lean_unsigned_to_nat(1289u); x_4 = lean_unsigned_to_nat(42u); x_5 = l_Lean_PrettyPrinter_Delaborator_delabFVar___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -54450,10 +51493,10 @@ l_Lean_getConstInfo___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__2_ lean_mark_persistent(l_Lean_getConstInfo___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__2___closed__3); l_Lean_getConstInfo___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__2___closed__4 = _init_l_Lean_getConstInfo___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__2___closed__4(); lean_mark_persistent(l_Lean_getConstInfo___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__2___closed__4); -l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__1 = _init_l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__1(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__1); -l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__2 = _init_l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__2(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__2); +l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__1 = _init_l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__1(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__1); +l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__2 = _init_l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__2(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__2); l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__19___closed__1 = _init_l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__19___closed__1(); lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__19___closed__1); l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__19___closed__2 = _init_l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__19___closed__2(); @@ -54792,6 +51835,8 @@ l_Lean_PrettyPrinter_Delaborator_delabOfNat___closed__5 = _init_l_Lean_PrettyPri lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_delabOfNat___closed__5); l_Lean_PrettyPrinter_Delaborator_delabOfNat___closed__6 = _init_l_Lean_PrettyPrinter_Delaborator_delabOfNat___closed__6(); lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_delabOfNat___closed__6); +l_Lean_PrettyPrinter_Delaborator_delabOfNat___closed__7 = _init_l_Lean_PrettyPrinter_Delaborator_delabOfNat___closed__7(); +lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_delabOfNat___closed__7); l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabOfNat__1___closed__1 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabOfNat__1___closed__1(); lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabOfNat__1___closed__1); l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabOfNat__1___closed__2 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabOfNat__1___closed__2(); @@ -54807,6 +51852,8 @@ lean_dec_ref(res); lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_delabNeg___closed__1); l_Lean_PrettyPrinter_Delaborator_delabNeg___closed__2 = _init_l_Lean_PrettyPrinter_Delaborator_delabNeg___closed__2(); lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_delabNeg___closed__2); +l_Lean_PrettyPrinter_Delaborator_delabNeg___closed__3 = _init_l_Lean_PrettyPrinter_Delaborator_delabNeg___closed__3(); +lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_delabNeg___closed__3); l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNeg__1___closed__1 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNeg__1___closed__1(); lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNeg__1___closed__1); l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNeg__1___closed__2 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNeg__1___closed__2(); @@ -54822,6 +51869,8 @@ lean_dec_ref(res); lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_delabHDiv___closed__1); l_Lean_PrettyPrinter_Delaborator_delabHDiv___closed__2 = _init_l_Lean_PrettyPrinter_Delaborator_delabHDiv___closed__2(); lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_delabHDiv___closed__2); +l_Lean_PrettyPrinter_Delaborator_delabHDiv___closed__3 = _init_l_Lean_PrettyPrinter_Delaborator_delabHDiv___closed__3(); +lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_delabHDiv___closed__3); l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabHDiv__1___closed__1 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabHDiv__1___closed__1(); lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabHDiv__1___closed__1); l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabHDiv__1___closed__2 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabHDiv__1___closed__2(); @@ -54851,6 +51900,8 @@ l_Lean_PrettyPrinter_Delaborator_delabOfScientific___closed__2 = _init_l_Lean_Pr lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_delabOfScientific___closed__2); l_Lean_PrettyPrinter_Delaborator_delabOfScientific___closed__3 = _init_l_Lean_PrettyPrinter_Delaborator_delabOfScientific___closed__3(); lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_delabOfScientific___closed__3); +l_Lean_PrettyPrinter_Delaborator_delabOfScientific___closed__4 = _init_l_Lean_PrettyPrinter_Delaborator_delabOfScientific___closed__4(); +lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_delabOfScientific___closed__4); l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabOfScientific__1___closed__1 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabOfScientific__1___closed__1(); lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabOfScientific__1___closed__1); l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabOfScientific__1___closed__2 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabOfScientific__1___closed__2(); @@ -54948,6 +51999,8 @@ l_Lean_PrettyPrinter_Delaborator_delabDIte___closed__2 = _init_l_Lean_PrettyPrin lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_delabDIte___closed__2); l_Lean_PrettyPrinter_Delaborator_delabDIte___closed__3 = _init_l_Lean_PrettyPrinter_Delaborator_delabDIte___closed__3(); lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_delabDIte___closed__3); +l_Lean_PrettyPrinter_Delaborator_delabDIte___closed__4 = _init_l_Lean_PrettyPrinter_Delaborator_delabDIte___closed__4(); +lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_delabDIte___closed__4); l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabDIte__1___closed__1 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabDIte__1___closed__1(); lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabDIte__1___closed__1); l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabDIte__1___closed__2 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabDIte__1___closed__2(); @@ -54973,6 +52026,8 @@ l_Lean_PrettyPrinter_Delaborator_delabCond___closed__2 = _init_l_Lean_PrettyPrin lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_delabCond___closed__2); l_Lean_PrettyPrinter_Delaborator_delabCond___closed__3 = _init_l_Lean_PrettyPrinter_Delaborator_delabCond___closed__3(); lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_delabCond___closed__3); +l_Lean_PrettyPrinter_Delaborator_delabCond___closed__4 = _init_l_Lean_PrettyPrinter_Delaborator_delabCond___closed__4(); +lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_delabCond___closed__4); l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabCond__1___closed__1 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabCond__1___closed__1(); lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabCond__1___closed__1); l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabCond__1___closed__2 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabCond__1___closed__2(); @@ -55139,6 +52194,8 @@ l_Lean_PrettyPrinter_Delaborator_delabDo___closed__1 = _init_l_Lean_PrettyPrinte lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_delabDo___closed__1); l_Lean_PrettyPrinter_Delaborator_delabDo___closed__2 = _init_l_Lean_PrettyPrinter_Delaborator_delabDo___closed__2(); lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_delabDo___closed__2); +l_Lean_PrettyPrinter_Delaborator_delabDo___closed__3 = _init_l_Lean_PrettyPrinter_Delaborator_delabDo___closed__3(); +lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_delabDo___closed__3); l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabDo__1___closed__1 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabDo__1___closed__1(); lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabDo__1___closed__1); l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabDo__1___closed__2 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabDo__1___closed__2(); @@ -55150,31 +52207,7 @@ lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabDo__1___ if (builtin) {res = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabDo__1(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1 = _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1(); -lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1); -l_Lean_PrettyPrinter_Delaborator_reifyName___closed__2 = _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__2(); -lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_reifyName___closed__2); -l_Lean_PrettyPrinter_Delaborator_reifyName___closed__3 = _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__3(); -lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_reifyName___closed__3); -l_Lean_PrettyPrinter_Delaborator_reifyName___closed__4 = _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__4(); -lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_reifyName___closed__4); -l_Lean_PrettyPrinter_Delaborator_reifyName___closed__5 = _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__5(); -lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_reifyName___closed__5); -l_Lean_PrettyPrinter_Delaborator_reifyName___closed__6 = _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__6(); -lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_reifyName___closed__6); -l_Lean_PrettyPrinter_Delaborator_reifyName___closed__7 = _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__7(); -lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_reifyName___closed__7); -l_Lean_PrettyPrinter_Delaborator_reifyName___closed__8 = _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__8(); -lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_reifyName___closed__8); -l_Lean_PrettyPrinter_Delaborator_reifyName___closed__9 = _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__9(); -lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_reifyName___closed__9); -l_Lean_PrettyPrinter_Delaborator_reifyName___closed__10 = _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__10(); -lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_reifyName___closed__10); -l_Lean_PrettyPrinter_Delaborator_reifyName___closed__11 = _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__11(); -lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_reifyName___closed__11); -l_Lean_PrettyPrinter_Delaborator_reifyName___closed__12 = _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__12(); -lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_reifyName___closed__12); -l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__1 = _init_l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__1(); +}l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__1 = _init_l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__1(); lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__1); l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__2 = _init_l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__2(); lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__2); @@ -55194,46 +52227,66 @@ l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__3 = _i lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__3); l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__4 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__4(); lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__4); +l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__5 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__5(); +lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__5); +l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__6 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__6(); +lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__6); if (builtin) {res = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__2___closed__1 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__2___closed__1(); lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__2___closed__1); +l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__2___closed__2 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__2___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__2___closed__2); if (builtin) {res = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__2(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__3___closed__1 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__3___closed__1(); lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__3___closed__1); +l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__3___closed__2 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__3___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__3___closed__2); if (builtin) {res = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__3(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__4___closed__1 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__4___closed__1(); lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__4___closed__1); +l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__4___closed__2 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__4___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__4___closed__2); if (builtin) {res = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__4(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__5___closed__1 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__5___closed__1(); lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__5___closed__1); +l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__5___closed__2 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__5___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__5___closed__2); if (builtin) {res = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__5(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__6___closed__1 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__6___closed__1(); lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__6___closed__1); +l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__6___closed__2 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__6___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__6___closed__2); if (builtin) {res = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__6(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__7___closed__1 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__7___closed__1(); lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__7___closed__1); +l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__7___closed__2 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__7___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__7___closed__2); if (builtin) {res = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__7(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__8___closed__1 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__8___closed__1(); lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__8___closed__1); +l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__8___closed__2 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__8___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__8___closed__2); if (builtin) {res = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__8(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__9___closed__1 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__9___closed__1(); lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__9___closed__1); +l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__9___closed__2 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__9___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__9___closed__2); if (builtin) {res = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__9(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); @@ -55245,6 +52298,8 @@ l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__3 = _i lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__3); l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__4 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__4(); lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__4); +l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__5 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__5(); +lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__5); if (builtin) {res = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Lean/PrettyPrinter/Delaborator/TopDownAnalyze.c b/stage0/stdlib/Lean/PrettyPrinter/Delaborator/TopDownAnalyze.c index 2418f3338be2..e122973cb1e3 100644 --- a/stage0/stdlib/Lean/PrettyPrinter/Delaborator/TopDownAnalyze.c +++ b/stage0/stdlib/Lean/PrettyPrinter/Delaborator/TopDownAnalyze.c @@ -29,6 +29,7 @@ static lean_object* l_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_analyze___cl LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_analyze_analyzeAppStaged___lambda__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_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_analyzeAppStagedCore_applyFunBinderHeuristic_core___spec__2___boxed(lean_object**); static lean_object* l_Lean_PrettyPrinter_Delaborator_initFn____x40_Lean_PrettyPrinter_Delaborator_TopDownAnalyze___hyg_10871____closed__12; +lean_object* l_Array_take___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_replaceLPsWithVars___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_PrettyPrinter_Delaborator_TopDownAnalyze___hyg_367_(lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_analyze_analyzeLet___spec__21(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -642,7 +643,6 @@ LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_PrettyPrinter_Delabora static lean_object* l_Lean_initFn____x40_Lean_PrettyPrinter_Delaborator_TopDownAnalyze___hyg_207____closed__1; LEAN_EXPORT uint8_t l_Lean_getPPAnalysisHole(lean_object*); static lean_object* l_Lean_initFn____x40_Lean_PrettyPrinter_Delaborator_TopDownAnalyze___hyg_287____closed__5; -lean_object* l_Array_shrink___rarg(lean_object*, lean_object*); lean_object* l_Lean_FindLevelMVar_main(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_withTraceNode___at_Lean_PrettyPrinter_Delaborator_topDownAnalyze___spec__2___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withNaryArg___at_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_analyzeAppStagedCore_analyzeArg___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*); @@ -27605,7 +27605,7 @@ x_25 = lean_array_get_size(x_22); lean_inc(x_25); x_26 = l_Array_extract___rarg(x_2, x_25, x_16); lean_dec(x_16); -x_27 = l_Array_shrink___rarg(x_2, x_25); +x_27 = l_Array_take___rarg(x_2, x_25); lean_dec(x_25); x_28 = lean_ctor_get_uint8(x_3, sizeof(void*)*1); if (x_28 == 0) diff --git a/stage0/stdlib/Lean/PrettyPrinter/Formatter.c b/stage0/stdlib/Lean/PrettyPrinter/Formatter.c index f1946137929b..3dd835e1a47d 100644 --- a/stage0/stdlib/Lean/PrettyPrinter/Formatter.c +++ b/stage0/stdlib/Lean/PrettyPrinter/Formatter.c @@ -29,6 +29,7 @@ LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Formatter_instCoeForallFormatterAl LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Formatter_instMonadTraverserFormatterM; static lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter_Formatter___hyg_5164____closed__3; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Formatter_pushToken___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Array_take___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Formatter_pushAlign(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Formatter_notFollowedBy_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter_Formatter___hyg_5647____closed__10; @@ -416,7 +417,6 @@ lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Formatter_charLitNoAntiquot_formatter___closed__2; static lean_object* l_Lean_PrettyPrinter_Formatter_pushToken___lambda__4___closed__4; lean_object* l_Lean_getConstInfo___at_Lean_registerInitAttrUnsafe___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Array_shrink___rarg(lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Formatter_categoryFormatterCore___closed__2; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Formatter_categoryFormatterCore___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_MonadTraverser_goLeft___at_Lean_PrettyPrinter_Formatter_visitArgs___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*); @@ -3157,7 +3157,7 @@ lean_inc(x_9); x_17 = l_Array_extract___rarg(x_14, x_9, x_16); lean_dec(x_16); x_18 = lean_apply_1(x_1, x_17); -x_19 = l_Array_shrink___rarg(x_14, x_9); +x_19 = l_Array_take___rarg(x_14, x_9); lean_dec(x_9); x_20 = lean_array_push(x_19, x_18); x_21 = l_Lean_PrettyPrinter_Formatter_setStack(x_20, x_3, x_4, x_5, x_6, x_15); diff --git a/stage0/stdlib/Lean/Server/CodeActions/Basic.c b/stage0/stdlib/Lean/Server/CodeActions/Basic.c index 091aef5554c0..a388116a38a6 100644 --- a/stage0/stdlib/Lean/Server/CodeActions/Basic.c +++ b/stage0/stdlib/Lean/Server/CodeActions/Basic.c @@ -92,6 +92,7 @@ LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Serve extern lean_object* l_Lean_Server_requestHandlers; lean_object* l_Lean_stringToMessageData(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_handleCodeActionResolve(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Server_handleCodeAction___spec__9___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_fromJsonCodeAction____x40_Lean_Data_Lsp_CodeActions___hyg_1204_(lean_object*); static lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_513____lambda__2___closed__6; LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_1540____spec__1___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); @@ -113,12 +114,12 @@ LEAN_EXPORT lean_object* l_Lean_Server_instFileSourceCodeAction(lean_object*); static lean_object* l_Lean_Server_CodeAction_getFileSource_x21___closed__4; size_t lean_usize_of_nat(lean_object*); extern lean_object* l_Lean_Server_instInhabitedRequestError; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Server_handleCodeAction___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_513____closed__25; static lean_object* l___private_Lean_Server_CodeActions_Basic_0__Lean_Server_fromJsonCodeActionResolveData____x40_Lean_Server_CodeActions_Basic___hyg_125____closed__1; static lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_1209____spec__2___closed__2; LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_1209____spec__3___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_FileMap_lspPosToUtf8Pos(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Server_handleCodeAction___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_1540____spec__1___lambda__2___closed__1; static lean_object* l_Lean_Server_instFromJsonCodeActionResolveData___closed__1; lean_object* lean_st_ref_take(lean_object*, lean_object*); @@ -162,6 +163,7 @@ lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); static lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_454____closed__4; LEAN_EXPORT lean_object* l_Lean_Server_handleCodeAction(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_513____closed__3; +lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_513____closed__26; static lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_513____closed__8; static lean_object* l___private_Lean_Server_CodeActions_Basic_0__Lean_Server_fromJsonCodeActionResolveData____x40_Lean_Server_CodeActions_Basic___hyg_125____closed__7; @@ -189,7 +191,6 @@ lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_ lean_object* l_Lean_registerSimplePersistentEnvExtension___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_handleCodeAction___spec__10(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ofExcept___at_Lean_Server_handleCodeAction___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); lean_object* l_Pi_instInhabited___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_codeActionProviderExt; static lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_513____lambda__3___closed__2; @@ -208,6 +209,7 @@ lean_object* l_Array_append___rarg(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_CodeActions_Basic_0__Lean_Server_fromJsonCodeActionResolveData____x40_Lean_Server_CodeActions_Basic___hyg_125____closed__18; LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_513____lambda__3(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_toJsonCodeActionParams____x40_Lean_Data_Lsp_CodeActions___hyg_612_(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Server_handleCodeAction___spec__9___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_513____lambda__5___closed__1; static lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_454____closed__1; static lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_513____lambda__2___closed__4; @@ -255,7 +257,6 @@ static lean_object* l___private_Lean_Server_CodeActions_Basic_0__Lean_Server_fro lean_object* l_Lean_registerBuiltinAttribute(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_513____lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_CodeActions_Basic_0__Lean_Server_fromJsonCodeActionResolveData____x40_Lean_Server_CodeActions_Basic___hyg_125____closed__12; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Server_handleCodeAction___spec__9___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l___private_Lean_Attributes_0__Lean_beqAttributeKind____x40_Lean_Attributes___hyg_162_(uint8_t, uint8_t); lean_object* l___private_Lean_ToExpr_0__Lean_Name_toExprAux(lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_revFold___at_Lean_Server_handleCodeAction___spec__7(lean_object*, lean_object*); @@ -277,17 +278,16 @@ LEAN_EXPORT lean_object* l_Lean_Server_handleCodeActionResolve___lambda__3(lean_ LEAN_EXPORT lean_object* l_Lean_Server_CodeAction_getFileSource_x21(lean_object*); static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_1209____spec__1___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Lean_Server_handleCodeAction___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Server_handleCodeAction___spec__9___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_513____lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_string_append(lean_object*, lean_object*); lean_object* l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_toJsonCodeAction____x40_Lean_Data_Lsp_CodeActions___hyg_1130_(lean_object*); uint8_t l_Lean_PersistentHashMap_contains___at_Lean_Server_registerLspRequestHandler___spec__6(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_1209_(lean_object*); LEAN_EXPORT lean_object* l_Lean_RBMap_toList___at_Lean_Server_handleCodeAction___spec__6(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Server_handleCodeAction___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_454____lambda__3(lean_object*); static lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_513____lambda__3___closed__1; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Server_handleCodeAction___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_513____lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -424,7 +424,7 @@ x_24 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_24, 0, x_7); lean_ctor_set(x_24, 1, x_23); x_25 = l___private_Lean_Server_CodeActions_Basic_0__Lean_Server_toJsonCodeActionResolveData____x40_Lean_Server_CodeActions_Basic___hyg_59____closed__5; -x_26 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_24, x_25); +x_26 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_24, x_25); x_27 = l_Lean_Json_mkObj(x_26); return x_27; } @@ -2588,7 +2588,7 @@ x_3 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Server_handleCodeActio return x_3; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Server_handleCodeAction___spec__9___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Server_handleCodeAction___spec__9___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; @@ -2656,7 +2656,7 @@ return x_26; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Server_handleCodeAction___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Server_handleCodeAction___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; uint8_t x_12; @@ -2694,7 +2694,7 @@ x_21 = lean_box(0); lean_inc(x_6); lean_inc(x_2); lean_inc(x_1); -x_22 = l_Array_mapIdxM_map___at_Lean_Server_handleCodeAction___spec__9___lambda__1(x_1, x_2, x_6, x_15, x_21, x_9, x_10); +x_22 = l_Array_mapFinIdxM_map___at_Lean_Server_handleCodeAction___spec__9___lambda__1(x_1, x_2, x_6, x_15, x_21, x_9, x_10); x_23 = lean_ctor_get(x_22, 0); lean_inc(x_23); x_24 = lean_ctor_get(x_22, 1); @@ -2755,7 +2755,7 @@ x_16 = lean_array_get_size(x_14); x_17 = lean_mk_empty_array_with_capacity(x_16); x_18 = lean_unsigned_to_nat(0u); lean_inc(x_1); -x_19 = l_Array_mapIdxM_map___at_Lean_Server_handleCodeAction___spec__9(x_1, x_11, x_14, x_14, x_16, x_18, lean_box(0), x_17, x_7, x_15); +x_19 = l_Array_mapFinIdxM_map___at_Lean_Server_handleCodeAction___spec__9(x_1, x_11, x_14, x_14, x_16, x_18, lean_box(0), x_17, x_7, x_15); lean_dec(x_14); x_20 = lean_ctor_get(x_19, 0); lean_inc(x_20); @@ -3288,21 +3288,21 @@ lean_dec(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Server_handleCodeAction___spec__9___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Server_handleCodeAction___spec__9___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; -x_8 = l_Array_mapIdxM_map___at_Lean_Server_handleCodeAction___spec__9___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Array_mapFinIdxM_map___at_Lean_Server_handleCodeAction___spec__9___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_6); lean_dec(x_5); return x_8; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Server_handleCodeAction___spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Server_handleCodeAction___spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; -x_11 = l_Array_mapIdxM_map___at_Lean_Server_handleCodeAction___spec__9(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Array_mapFinIdxM_map___at_Lean_Server_handleCodeAction___spec__9(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_9); lean_dec(x_4); lean_dec(x_3); diff --git a/stage0/stdlib/Lean/Server/Completion.c b/stage0/stdlib/Lean/Server/Completion.c index 6c70fea7af8d..71ac5113cacd 100644 --- a/stage0/stdlib/Lean/Server/Completion.c +++ b/stage0/stdlib/Lean/Server/Completion.c @@ -23,7 +23,6 @@ lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_forIn___at___private_Lean_Server_Completion_0__Lean_Server_Completion_idCompletionCore___spec__24(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_foldlM___at_Lean_Server_Completion_completeNamespaces___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_string_utf8_extract(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_CompletionItem_resolve___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Completion_completeNamespaces___spec__9(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_ppExpr(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -45,6 +44,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Lsp_toJsonCo LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_matchDecl_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_isDefEqToAppOf___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_addUnresolvedCompletionItem(lean_object*, lean_object*, uint8_t, double, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_dotIdCompletion___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_forEligibleDeclsM___spec__3(lean_object*); @@ -62,11 +62,11 @@ LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Compl LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_dotIdCompletion___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_foldlMAux_traverse___at_Lean_Server_Completion_completeNamespaces___spec__8___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Server_Completion_0__Lean_Server_Completion_isSyntheticTacticCompletion_isCompletionOnTacticBlockIndentation(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__3; static lean_object* l___private_Lean_Server_Completion_0__Lean_Lsp_fromJsonCompletionIdentifier____x40_Lean_Server_Completion___hyg_136____lambda__3___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_addNamespaceCompletionItem___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_private_to_user_name(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_fieldIdCompletion___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_findCompletionInfoAt_x3f_choose___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_getIndentationAmount___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Json_mkObj(lean_object*); @@ -141,11 +141,11 @@ LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Compl LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_dotCompletion___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_ConstantInfo_name(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_idCompletionCore___spec__23(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__1; static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_findSyntheticIdentifierCompletion_x3f___lambda__3___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_isDefEqToAppOf___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_getDotCompletionTypeNames_visit___spec__3(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_fvarId_x21(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_environment_find(lean_object*, lean_object*); @@ -153,7 +153,7 @@ uint8_t lean_float_decLt(double, double); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f_choose___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_addUnresolvedCompletionItem___lambda__2___closed__1; static lean_object* l_Lean_Server_Completion_getEligibleHeaderDecls___closed__2; -static lean_object* l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__4; +LEAN_EXPORT lean_object* l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_forEligibleDeclsM___spec__4(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_findSyntheticIdentifierCompletion_x3f___lambda__2___boxed(lean_object*); static lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Server_Completion_0__Lean_Server_Completion_isSyntheticTacticCompletion_isCompletionAfterSemicolon___spec__1___closed__1; @@ -165,7 +165,7 @@ LEAN_EXPORT lean_object* l_Lean_isEnumType___at___private_Lean_Server_Completion LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Lsp_toJsonCompletionIdentifier____x40_Lean_Server_Completion___hyg_270_(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_findSomeMAux___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findOutermostContextInfo_x3f_go___spec__2___boxed(lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_addKeywordCompletionItem___closed__3; -LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___rarg___lambda__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___rarg___lambda__1(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_InfoTree_foldInfo___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Completion_completeNamespaces___lambda__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Lsp_fromJsonCompletionIdentifier____x40_Lean_Server_Completion___hyg_136_(lean_object*); @@ -175,7 +175,6 @@ extern lean_object* l_Lean_instInhabitedJson; static lean_object* l___private_Lean_Server_Completion_0__Lean_Lsp_fromJsonCompletionIdentifier____x40_Lean_Server_Completion___hyg_136____lambda__1___closed__2; uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_optionCompletion___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Nat_nextPowerOfTwo_go(lean_object*, lean_object*, lean_object*); lean_object* lean_string_utf8_set(lean_object*, lean_object*, uint32_t); lean_object* l_Lean_Expr_cleanupAnnotations(lean_object*); @@ -207,15 +206,14 @@ LEAN_EXPORT lean_object* l_ReaderT_bind___at___private_Lean_Server_Completion_0_ LEAN_EXPORT lean_object* l_Lean_Server_Completion_completeNamespaces___lambda__1(uint8_t, lean_object*, lean_object*, lean_object*, double, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Server_Completion_0__Lean_Server_Completion_isSyntheticTacticCompletion_isCompletionOnTacticBlockIndentation___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_addUnresolvedCompletionItemForDecl(lean_object*, lean_object*, double, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__8; static double l___private_Lean_Server_Completion_0__Lean_Server_Completion_matchAtomic___closed__1; static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_dotCompletion___lambda__6___closed__2; extern lean_object* l_instInhabitedNat; -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1(lean_object*); lean_object* l_Lean_Parser_getTokenTable(lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Server_Completion_completeNamespaces___spec__1___closed__2; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_idCompletionCore___spec__14___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_idCompletionCore___lambda__3___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2(lean_object*); lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Server_CompletionItemData_0__Lean_Lsp_fromJsonCompletionItemData____x40_Lean_Server_CompletionItemData___hyg_15____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_insert___at___private_Lean_Server_Completion_0__Lean_Server_Completion_getDotCompletionTypeNames_visit___spec__1(lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_projectionFnInfoExt; @@ -227,7 +225,6 @@ LEAN_EXPORT lean_object* l_Lean_RBNode_ins___at___private_Lean_Server_Completion LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findOutermostContextInfo_x3f_go___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_dotIdCompletion___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Lsp_fromJsonCompletionItemDataWithId____x40_Lean_Server_Completion___hyg_366____closed__2; -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_truncate_go(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_getDotCompletionTypeNames(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Server_Completion_0__Lean_Server_Completion_allowCompletion(lean_object*, lean_object*, lean_object*); @@ -255,7 +252,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Compl LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_idCompletionCore___spec__17___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Server_Completion_0__Lean_Server_Completion_isSyntheticTacticCompletion_isEmpty(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_isDotCompletionMethod___spec__1(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_foldlMAux_traverse___at___private_Lean_Server_Completion_0__Lean_Server_Completion_idCompletionCore___spec__15(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonCompletionItemDataWithId; LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_forEligibleDeclsM___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*); @@ -267,6 +263,7 @@ lean_object* l_Lean_Elab_Info_tailPos_x3f(lean_object*); uint8_t l_List_elem___at_Lean_addAliasEntry___spec__16(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_tacticCompletion___spec__1___boxed__const__1; LEAN_EXPORT uint8_t l___private_Lean_Server_Completion_0__Lean_Server_Completion_isSyntheticTacticCompletion_isCompletionInEmptyTacticBlock(lean_object*, lean_object*, lean_object*); +uint8_t l_Lean_ConstantInfo_isTheorem(lean_object*); lean_object* lean_local_ctx_find(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_qsort_sort___at___private_Lean_Server_Completion_0__Lean_Server_Completion_sortCompletionItems___spec__2___lambda__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Lsp_fromJsonCompletionIdentifier____x40_Lean_Server_Completion___hyg_136____lambda__3___closed__2; @@ -319,6 +316,7 @@ lean_object* l_Lean_Name_getPrefix(lean_object*); lean_object* l_Lean_Elab_PartialContextInfo_mergeIntoOuter_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at___private_Lean_Server_Completion_0__Lean_Server_Completion_dotCompletion___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_ConstantInfo_isCtor(lean_object*); +LEAN_EXPORT lean_object* l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2(lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__5; static lean_object* l___private_Lean_Server_Completion_0__Lean_Lsp_fromJsonCompletionIdentifier____x40_Lean_Server_Completion___hyg_136____closed__6; LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_addKeywordCompletionItem___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -346,6 +344,7 @@ LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonCompletionIdentifier; static lean_object* l___private_Lean_Server_Completion_0__Lean_Lsp_fromJsonCompletionItemDataWithId____x40_Lean_Server_Completion___hyg_366____closed__11; LEAN_EXPORT lean_object* l_Lean_Lsp_CompletionItem_resolve___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_forEligibleDeclsM___spec__4___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_idCompletionCore(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_idCompletionCore___spec__26___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -373,6 +372,7 @@ lean_object* l_Lean_Name_append(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f_choose___spec__1___rarg(lean_object*, lean_object*); lean_object* l_Lean_Syntax_getTrailingSize(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts(lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); uint8_t lean_string_utf8_at_end(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Lsp_fromJsonCompletionItemDataWithId____x40_Lean_Server_Completion___hyg_366____closed__15; static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_addNamespaceCompletionItem___closed__3; @@ -426,13 +426,11 @@ LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_foldlMAux_traverse___at_Lean_S LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_dotCompletion___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Lsp_fromJsonCompletionIdentifier____x40_Lean_Server_Completion___hyg_136____lambda__3___closed__5; LEAN_EXPORT uint8_t l___private_Lean_Server_Completion_0__Lean_Server_Completion_findSyntheticIdentifierCompletion_x3f___lambda__2(lean_object*); -static lean_object* l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_normPrivateName_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_addNamespaceCompletionItem(lean_object*, double, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_CompletionItem_resolve(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_idCompletionCore___spec__1___lambda__1(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_isIdent(lean_object*); -lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Server_Completion_0__Lean_Server_Completion_isSyntheticTacticCompletion_isCompletionAfterSemicolon(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_fvarId(lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Lsp_fromJsonCompletionIdentifier____x40_Lean_Server_Completion___hyg_136____lambda__3___closed__8; @@ -461,7 +459,6 @@ extern lean_object* l_Lean_instInhabitedProjectionFunctionInfo; LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_truncate(lean_object*, lean_object*); uint8_t l_Lean_Environment_contains(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f_choose___spec__1(lean_object*); lean_object* l_Lean_MessageData_ofExpr(lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_isSyntheticTacticCompletion_isEmptyTacticBlock___closed__1; @@ -482,7 +479,6 @@ LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_foldlMAux_traverse___at___priv static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_isSyntheticTacticCompletion_getTacticsNode_x3f___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_idCompletionCore___lambda__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_isSyntheticTacticCompletion_go___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__4(lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Lsp_fromJsonCompletionIdentifier____x40_Lean_Server_Completion___hyg_136____lambda__3___closed__9; LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_dotCompletion___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Completion_completeNamespaces(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -509,6 +505,7 @@ static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion static lean_object* l___private_Lean_Server_Completion_0__Lean_Lsp_fromJsonCompletionItemDataWithId____x40_Lean_Server_Completion___hyg_366____closed__7; LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_dotIdCompletion___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Lsp_fromJsonCompletionIdentifier____x40_Lean_Server_Completion___hyg_136____lambda__1(lean_object*); +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__3; LEAN_EXPORT uint8_t l___private_Lean_Server_Completion_0__Lean_Server_Completion_findClosestInfoWithLocalContextAt_x3f_isBetter(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_idCompletionCore___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_isDotIdCompletionMethod___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -556,8 +553,6 @@ static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_getDotCompletionTypeNames_visit___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_findSyntheticIdentifierCompletion_x3f___lambda__5___closed__1; lean_object* l_Lean_ParametricAttribute_getParam_x3f___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__4___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findOutermostContextInfo_x3f_go___spec__5(lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_findSyntheticIdentifierCompletion_x3f___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_idCompletionCore___spec__16(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -607,6 +602,7 @@ uint8_t l_Lean_Expr_isProp(lean_object*); lean_object* lean_nat_mul(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_fieldIdCompletion___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_getDotCompletionTypeNames_visit___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_dotCompletion___lambda__6___closed__1; lean_object* l_Lean_Syntax_getRange_x3f(lean_object*, uint8_t); @@ -644,7 +640,6 @@ lean_object* l_Lean_instantiateMVarsCore(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_isDotCompletionMethod___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_truncate_go___closed__2; lean_object* l_List_dropWhile___rarg(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__2; lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_SynthInstance_removeUnusedArguments_x3f___spec__2___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_getIndentationAmount___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_optionCompletion___closed__4; @@ -711,6 +706,7 @@ static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_idCompletionCore___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_isSyntheticTacticCompletion_go___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_findSomeM_x3f___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findOutermostContextInfo_x3f_go___spec__1___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_dotIdCompletion___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); @@ -751,7 +747,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Compl uint8_t l_Lean_Name_isInternal(lean_object*); LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Server_Completion_0__Lean_Lsp_toJsonCompletionItemDataWithId____x40_Lean_Server_Completion___hyg_472____spec__1(lean_object*, lean_object*); lean_object* lean_array_uset(lean_object*, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonCompletionIdentifier; uint8_t lean_local_ctx_is_empty(lean_object*); lean_object* lean_expr_instantiate1(lean_object*, lean_object*); @@ -759,21 +754,23 @@ lean_object* l___private_Init_Data_Repr_0__Nat_reprFast(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Completion_getEligibleHeaderDecls___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Lsp_CompletionItem_resolve___closed__2; lean_object* l_Lean_Elab_ContextInfo_runMetaM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3___rarg(lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_addUnresolvedCompletionItem___lambda__2___closed__3; static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_dotCompletion___lambda__6___closed__3; LEAN_EXPORT lean_object* l_Lean_Server_Completion_completeNamespaces___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_allowCompletion___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__2; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_idCompletionCore___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_SMap_forM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_idCompletionCore___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_forEligibleDeclsM___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_land(size_t, size_t); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_findSyntheticIdentifierCompletion_x3f___lambda__3___boxed(lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Lsp_fromJsonCompletionIdentifier____x40_Lean_Server_Completion___hyg_136____closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1(lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_fieldIdCompletion___closed__1; static lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Server_Completion_0__Lean_Server_Completion_optionCompletion___spec__1___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_findClosestInfoWithLocalContextAt_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_matchDecl_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_findSyntheticIdentifierCompletion_x3f___lambda__5___closed__3; lean_object* lean_data_value_to_string(lean_object*); @@ -2215,7 +2212,7 @@ x_12 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_12, 0, x_7); lean_ctor_set(x_12, 1, x_11); x_13 = l___private_Lean_Server_Completion_0__Lean_Lsp_toJsonCompletionItemDataWithId____x40_Lean_Server_Completion___hyg_472____closed__1; -x_14 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); +x_14 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); x_15 = l_Lean_Json_mkObj(x_14); return x_15; } @@ -5527,7 +5524,7 @@ static lean_object* _init_l___private_Lean_Server_Completion_0__Lean_Server_Comp _start: { uint8_t x_1; lean_object* x_2; lean_object* x_3; -x_1 = 21; +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); @@ -5538,7 +5535,7 @@ static lean_object* _init_l___private_Lean_Server_Completion_0__Lean_Server_Comp _start: { uint8_t x_1; lean_object* x_2; lean_object* x_3; -x_1 = 12; +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); @@ -5549,7 +5546,7 @@ static lean_object* _init_l___private_Lean_Server_Completion_0__Lean_Server_Comp _start: { uint8_t x_1; lean_object* x_2; lean_object* x_3; -x_1 = 6; +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); @@ -5560,6 +5557,17 @@ static lean_object* _init_l___private_Lean_Server_Completion_0__Lean_Server_Comp _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; +} +} +static lean_object* _init_l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__8() { +_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); @@ -5588,522 +5596,556 @@ uint8_t x_15; x_15 = l_Lean_ConstantInfo_isInductive(x_1); if (x_15 == 0) { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; +uint8_t x_16; lean_dec(x_13); +x_16 = l_Lean_ConstantInfo_isTheorem(x_1); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; lean_free_object(x_9); -x_16 = l_Lean_ConstantInfo_name(x_1); -x_17 = l_Lean_isProjectionFn___at___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___spec__1(x_16, x_2, x_3, x_4, x_5, x_6, x_7, x_12); -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); +x_17 = l_Lean_ConstantInfo_name(x_1); +x_18 = l_Lean_isProjectionFn___at___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___spec__1(x_17, x_2, x_3, x_4, x_5, x_6, x_7, x_12); x_19 = lean_ctor_get(x_18, 0); lean_inc(x_19); -lean_dec(x_18); -x_20 = lean_unbox(x_19); +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); lean_dec(x_19); -if (x_20 == 0) +x_21 = lean_unbox(x_20); +lean_dec(x_20); +if (x_21 == 0) { -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_17, 1); -lean_inc(x_21); -lean_dec(x_17); -x_22 = l_Lean_ConstantInfo_type(x_1); -x_23 = lean_whnf(x_22, x_4, x_5, x_6, x_7, x_21); -if (lean_obj_tag(x_23) == 0) +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 = l_Lean_ConstantInfo_type(x_1); +x_24 = lean_whnf(x_23, x_4, x_5, x_6, x_7, x_22); +if (lean_obj_tag(x_24) == 0) { -uint8_t x_24; -x_24 = !lean_is_exclusive(x_23); -if (x_24 == 0) +uint8_t x_25; +x_25 = !lean_is_exclusive(x_24); +if (x_25 == 0) { -lean_object* x_25; uint8_t x_26; -x_25 = lean_ctor_get(x_23, 0); -x_26 = l_Lean_Expr_isForall(x_25); -lean_dec(x_25); -if (x_26 == 0) +lean_object* x_26; uint8_t x_27; +x_26 = lean_ctor_get(x_24, 0); +x_27 = l_Lean_Expr_isForall(x_26); +lean_dec(x_26); +if (x_27 == 0) { -lean_object* x_27; -x_27 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__1; -lean_ctor_set(x_23, 0, x_27); -return x_23; +lean_object* x_28; +x_28 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__1; +lean_ctor_set(x_24, 0, x_28); +return x_24; } else { -lean_object* x_28; -x_28 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__2; -lean_ctor_set(x_23, 0, x_28); -return x_23; +lean_object* x_29; +x_29 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__2; +lean_ctor_set(x_24, 0, x_29); +return x_24; } } else { -lean_object* x_29; lean_object* x_30; uint8_t x_31; -x_29 = lean_ctor_get(x_23, 0); -x_30 = lean_ctor_get(x_23, 1); +lean_object* x_30; lean_object* x_31; uint8_t x_32; +x_30 = lean_ctor_get(x_24, 0); +x_31 = lean_ctor_get(x_24, 1); +lean_inc(x_31); lean_inc(x_30); -lean_inc(x_29); -lean_dec(x_23); -x_31 = l_Lean_Expr_isForall(x_29); -lean_dec(x_29); -if (x_31 == 0) +lean_dec(x_24); +x_32 = l_Lean_Expr_isForall(x_30); +lean_dec(x_30); +if (x_32 == 0) { -lean_object* x_32; lean_object* x_33; -x_32 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___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_30); -return x_33; +lean_object* x_33; lean_object* x_34; +x_33 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__1; +x_34 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_34, 0, x_33); +lean_ctor_set(x_34, 1, x_31); +return x_34; } else { -lean_object* x_34; lean_object* x_35; -x_34 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__2; -x_35 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_35, 0, x_34); -lean_ctor_set(x_35, 1, x_30); -return x_35; +lean_object* x_35; lean_object* x_36; +x_35 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__2; +x_36 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_36, 0, x_35); +lean_ctor_set(x_36, 1, x_31); +return x_36; } } } else { -uint8_t x_36; -x_36 = !lean_is_exclusive(x_23); -if (x_36 == 0) +uint8_t x_37; +x_37 = !lean_is_exclusive(x_24); +if (x_37 == 0) { -return x_23; +return x_24; } else { -lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_37 = lean_ctor_get(x_23, 0); -x_38 = lean_ctor_get(x_23, 1); +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_24, 0); +x_39 = lean_ctor_get(x_24, 1); +lean_inc(x_39); lean_inc(x_38); -lean_inc(x_37); -lean_dec(x_23); -x_39 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_39, 0, x_37); -lean_ctor_set(x_39, 1, x_38); -return x_39; +lean_dec(x_24); +x_40 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +return x_40; } } } else { -uint8_t x_40; +uint8_t x_41; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_40 = !lean_is_exclusive(x_17); -if (x_40 == 0) +x_41 = !lean_is_exclusive(x_18); +if (x_41 == 0) { -lean_object* x_41; lean_object* x_42; -x_41 = lean_ctor_get(x_17, 0); -lean_dec(x_41); -x_42 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__3; -lean_ctor_set(x_17, 0, x_42); -return x_17; +lean_object* x_42; lean_object* x_43; +x_42 = lean_ctor_get(x_18, 0); +lean_dec(x_42); +x_43 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__3; +lean_ctor_set(x_18, 0, x_43); +return x_18; } else { -lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_43 = lean_ctor_get(x_17, 1); -lean_inc(x_43); -lean_dec(x_17); -x_44 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__3; -x_45 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_45, 0, x_44); -lean_ctor_set(x_45, 1, x_43); -return x_45; +lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_44 = lean_ctor_get(x_18, 1); +lean_inc(x_44); +lean_dec(x_18); +x_45 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___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_44); +return x_46; } } } else { -lean_object* x_46; uint8_t x_47; -x_46 = l_Lean_ConstantInfo_name(x_1); -lean_inc(x_46); -x_47 = lean_is_class(x_13, x_46); -if (x_47 == 0) +lean_object* x_47; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_47 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__4; +lean_ctor_set(x_9, 0, x_47); +return x_9; +} +} +else { -lean_object* x_48; +lean_object* x_48; uint8_t x_49; +x_48 = l_Lean_ConstantInfo_name(x_1); +lean_inc(x_48); +x_49 = lean_is_class(x_13, x_48); +if (x_49 == 0) +{ +lean_object* x_50; lean_free_object(x_9); -x_48 = l_Lean_isEnumType___at___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___spec__2(x_46, x_2, x_3, x_4, x_5, x_6, x_7, x_12); +x_50 = l_Lean_isEnumType___at___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___spec__2(x_48, 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); -if (lean_obj_tag(x_48) == 0) +if (lean_obj_tag(x_50) == 0) { -lean_object* x_49; lean_object* x_50; uint8_t x_51; -x_49 = lean_ctor_get(x_48, 0); -lean_inc(x_49); -x_50 = lean_ctor_get(x_49, 0); -lean_inc(x_50); -lean_dec(x_49); -x_51 = lean_unbox(x_50); -lean_dec(x_50); -if (x_51 == 0) +lean_object* x_51; lean_object* x_52; uint8_t x_53; +x_51 = lean_ctor_get(x_50, 0); +lean_inc(x_51); +x_52 = lean_ctor_get(x_51, 0); +lean_inc(x_52); +lean_dec(x_51); +x_53 = lean_unbox(x_52); +lean_dec(x_52); +if (x_53 == 0) { -uint8_t x_52; -x_52 = !lean_is_exclusive(x_48); -if (x_52 == 0) +uint8_t x_54; +x_54 = !lean_is_exclusive(x_50); +if (x_54 == 0) { -lean_object* x_53; lean_object* x_54; -x_53 = lean_ctor_get(x_48, 0); -lean_dec(x_53); -x_54 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__4; -lean_ctor_set(x_48, 0, x_54); -return x_48; +lean_object* x_55; lean_object* x_56; +x_55 = lean_ctor_get(x_50, 0); +lean_dec(x_55); +x_56 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__5; +lean_ctor_set(x_50, 0, x_56); +return x_50; } else { -lean_object* x_55; lean_object* x_56; lean_object* x_57; -x_55 = lean_ctor_get(x_48, 1); -lean_inc(x_55); -lean_dec(x_48); -x_56 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__4; -x_57 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_57, 0, x_56); -lean_ctor_set(x_57, 1, x_55); -return x_57; +lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_57 = lean_ctor_get(x_50, 1); +lean_inc(x_57); +lean_dec(x_50); +x_58 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__5; +x_59 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_59, 0, x_58); +lean_ctor_set(x_59, 1, x_57); +return x_59; } } else { -uint8_t x_58; -x_58 = !lean_is_exclusive(x_48); -if (x_58 == 0) +uint8_t x_60; +x_60 = !lean_is_exclusive(x_50); +if (x_60 == 0) { -lean_object* x_59; lean_object* x_60; -x_59 = lean_ctor_get(x_48, 0); -lean_dec(x_59); -x_60 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__5; -lean_ctor_set(x_48, 0, x_60); -return x_48; +lean_object* x_61; lean_object* x_62; +x_61 = lean_ctor_get(x_50, 0); +lean_dec(x_61); +x_62 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__6; +lean_ctor_set(x_50, 0, x_62); +return x_50; } else { -lean_object* x_61; lean_object* x_62; lean_object* x_63; -x_61 = lean_ctor_get(x_48, 1); -lean_inc(x_61); -lean_dec(x_48); -x_62 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__5; -x_63 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_63, 0, x_62); -lean_ctor_set(x_63, 1, x_61); -return x_63; +lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_63 = lean_ctor_get(x_50, 1); +lean_inc(x_63); +lean_dec(x_50); +x_64 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__6; +x_65 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_65, 0, x_64); +lean_ctor_set(x_65, 1, x_63); +return x_65; } } } else { -uint8_t x_64; -x_64 = !lean_is_exclusive(x_48); -if (x_64 == 0) +uint8_t x_66; +x_66 = !lean_is_exclusive(x_50); +if (x_66 == 0) { -return x_48; +return x_50; } else { -lean_object* x_65; lean_object* x_66; lean_object* x_67; -x_65 = lean_ctor_get(x_48, 0); -x_66 = lean_ctor_get(x_48, 1); -lean_inc(x_66); -lean_inc(x_65); -lean_dec(x_48); -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_67; lean_object* x_68; lean_object* x_69; +x_67 = lean_ctor_get(x_50, 0); +x_68 = lean_ctor_get(x_50, 1); +lean_inc(x_68); +lean_inc(x_67); +lean_dec(x_50); +x_69 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_69, 0, x_67); +lean_ctor_set(x_69, 1, x_68); +return x_69; } } } else { -lean_object* x_68; -lean_dec(x_46); +lean_object* x_70; +lean_dec(x_48); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_68 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__6; -lean_ctor_set(x_9, 0, x_68); +x_70 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__7; +lean_ctor_set(x_9, 0, x_70); return x_9; } } } else { -lean_object* x_69; +lean_object* x_71; lean_dec(x_13); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_69 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__7; -lean_ctor_set(x_9, 0, x_69); +x_71 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__8; +lean_ctor_set(x_9, 0, x_71); return x_9; } } else { -lean_object* x_70; lean_object* x_71; lean_object* x_72; uint8_t x_73; -x_70 = lean_ctor_get(x_9, 0); -x_71 = lean_ctor_get(x_9, 1); -lean_inc(x_71); -lean_inc(x_70); -lean_dec(x_9); -x_72 = lean_ctor_get(x_70, 0); +lean_object* x_72; lean_object* x_73; lean_object* x_74; uint8_t x_75; +x_72 = lean_ctor_get(x_9, 0); +x_73 = lean_ctor_get(x_9, 1); +lean_inc(x_73); lean_inc(x_72); -lean_dec(x_70); -x_73 = l_Lean_ConstantInfo_isCtor(x_1); -if (x_73 == 0) +lean_dec(x_9); +x_74 = lean_ctor_get(x_72, 0); +lean_inc(x_74); +lean_dec(x_72); +x_75 = l_Lean_ConstantInfo_isCtor(x_1); +if (x_75 == 0) { -uint8_t x_74; -x_74 = l_Lean_ConstantInfo_isInductive(x_1); -if (x_74 == 0) +uint8_t x_76; +x_76 = l_Lean_ConstantInfo_isInductive(x_1); +if (x_76 == 0) { -lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; uint8_t x_79; -lean_dec(x_72); -x_75 = l_Lean_ConstantInfo_name(x_1); -x_76 = l_Lean_isProjectionFn___at___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___spec__1(x_75, x_2, x_3, x_4, x_5, x_6, x_7, x_71); -x_77 = lean_ctor_get(x_76, 0); -lean_inc(x_77); -x_78 = lean_ctor_get(x_77, 0); -lean_inc(x_78); -lean_dec(x_77); -x_79 = lean_unbox(x_78); -lean_dec(x_78); -if (x_79 == 0) +uint8_t x_77; +lean_dec(x_74); +x_77 = l_Lean_ConstantInfo_isTheorem(x_1); +if (x_77 == 0) { -lean_object* x_80; lean_object* x_81; lean_object* x_82; -x_80 = lean_ctor_get(x_76, 1); +lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; uint8_t x_82; +x_78 = l_Lean_ConstantInfo_name(x_1); +x_79 = l_Lean_isProjectionFn___at___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___spec__1(x_78, x_2, x_3, x_4, x_5, x_6, x_7, x_73); +x_80 = lean_ctor_get(x_79, 0); lean_inc(x_80); -lean_dec(x_76); -x_81 = l_Lean_ConstantInfo_type(x_1); -x_82 = lean_whnf(x_81, x_4, x_5, x_6, x_7, x_80); -if (lean_obj_tag(x_82) == 0) +x_81 = lean_ctor_get(x_80, 0); +lean_inc(x_81); +lean_dec(x_80); +x_82 = lean_unbox(x_81); +lean_dec(x_81); +if (x_82 == 0) { -lean_object* x_83; lean_object* x_84; lean_object* x_85; uint8_t x_86; -x_83 = lean_ctor_get(x_82, 0); +lean_object* x_83; lean_object* x_84; lean_object* x_85; +x_83 = lean_ctor_get(x_79, 1); lean_inc(x_83); -x_84 = lean_ctor_get(x_82, 1); -lean_inc(x_84); -if (lean_is_exclusive(x_82)) { - lean_ctor_release(x_82, 0); - lean_ctor_release(x_82, 1); - x_85 = x_82; +lean_dec(x_79); +x_84 = l_Lean_ConstantInfo_type(x_1); +x_85 = lean_whnf(x_84, x_4, x_5, x_6, x_7, x_83); +if (lean_obj_tag(x_85) == 0) +{ +lean_object* x_86; lean_object* x_87; lean_object* x_88; uint8_t 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); +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_82); - x_85 = lean_box(0); + lean_dec_ref(x_85); + x_88 = lean_box(0); } -x_86 = l_Lean_Expr_isForall(x_83); -lean_dec(x_83); -if (x_86 == 0) +x_89 = l_Lean_Expr_isForall(x_86); +lean_dec(x_86); +if (x_89 == 0) { -lean_object* x_87; lean_object* x_88; -x_87 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__1; -if (lean_is_scalar(x_85)) { - x_88 = lean_alloc_ctor(0, 2, 0); +lean_object* x_90; lean_object* x_91; +x_90 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__1; +if (lean_is_scalar(x_88)) { + x_91 = lean_alloc_ctor(0, 2, 0); } else { - x_88 = x_85; + x_91 = x_88; } -lean_ctor_set(x_88, 0, x_87); -lean_ctor_set(x_88, 1, x_84); -return x_88; +lean_ctor_set(x_91, 0, x_90); +lean_ctor_set(x_91, 1, x_87); +return x_91; } else { -lean_object* x_89; lean_object* x_90; -x_89 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__2; -if (lean_is_scalar(x_85)) { - x_90 = lean_alloc_ctor(0, 2, 0); +lean_object* x_92; lean_object* x_93; +x_92 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__2; +if (lean_is_scalar(x_88)) { + x_93 = lean_alloc_ctor(0, 2, 0); } else { - x_90 = x_85; + x_93 = x_88; } -lean_ctor_set(x_90, 0, x_89); -lean_ctor_set(x_90, 1, x_84); -return x_90; +lean_ctor_set(x_93, 0, x_92); +lean_ctor_set(x_93, 1, x_87); +return x_93; } } else { -lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; -x_91 = lean_ctor_get(x_82, 0); -lean_inc(x_91); -x_92 = lean_ctor_get(x_82, 1); -lean_inc(x_92); -if (lean_is_exclusive(x_82)) { - lean_ctor_release(x_82, 0); - lean_ctor_release(x_82, 1); - x_93 = x_82; +lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; +x_94 = lean_ctor_get(x_85, 0); +lean_inc(x_94); +x_95 = lean_ctor_get(x_85, 1); +lean_inc(x_95); +if (lean_is_exclusive(x_85)) { + lean_ctor_release(x_85, 0); + lean_ctor_release(x_85, 1); + x_96 = x_85; } else { - lean_dec_ref(x_82); - x_93 = lean_box(0); + lean_dec_ref(x_85); + x_96 = lean_box(0); } -if (lean_is_scalar(x_93)) { - x_94 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_96)) { + x_97 = lean_alloc_ctor(1, 2, 0); } else { - x_94 = x_93; + x_97 = x_96; } -lean_ctor_set(x_94, 0, x_91); -lean_ctor_set(x_94, 1, x_92); -return x_94; +lean_ctor_set(x_97, 0, x_94); +lean_ctor_set(x_97, 1, x_95); +return x_97; } } else { -lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; +lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_95 = lean_ctor_get(x_76, 1); -lean_inc(x_95); -if (lean_is_exclusive(x_76)) { - lean_ctor_release(x_76, 0); - lean_ctor_release(x_76, 1); - x_96 = x_76; +x_98 = lean_ctor_get(x_79, 1); +lean_inc(x_98); +if (lean_is_exclusive(x_79)) { + lean_ctor_release(x_79, 0); + lean_ctor_release(x_79, 1); + x_99 = x_79; } else { - lean_dec_ref(x_76); - x_96 = lean_box(0); + lean_dec_ref(x_79); + x_99 = lean_box(0); } -x_97 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__3; -if (lean_is_scalar(x_96)) { - x_98 = lean_alloc_ctor(0, 2, 0); +x_100 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__3; +if (lean_is_scalar(x_99)) { + x_101 = lean_alloc_ctor(0, 2, 0); } else { - x_98 = x_96; + x_101 = x_99; } -lean_ctor_set(x_98, 0, x_97); -lean_ctor_set(x_98, 1, x_95); -return x_98; +lean_ctor_set(x_101, 0, x_100); +lean_ctor_set(x_101, 1, x_98); +return x_101; } } else { -lean_object* x_99; uint8_t x_100; -x_99 = l_Lean_ConstantInfo_name(x_1); -lean_inc(x_99); -x_100 = lean_is_class(x_72, x_99); -if (x_100 == 0) +lean_object* x_102; lean_object* x_103; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_102 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__4; +x_103 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_103, 0, x_102); +lean_ctor_set(x_103, 1, x_73); +return x_103; +} +} +else { -lean_object* x_101; -x_101 = l_Lean_isEnumType___at___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___spec__2(x_99, x_2, x_3, x_4, x_5, x_6, x_7, x_71); +lean_object* x_104; uint8_t x_105; +x_104 = l_Lean_ConstantInfo_name(x_1); +lean_inc(x_104); +x_105 = lean_is_class(x_74, x_104); +if (x_105 == 0) +{ +lean_object* x_106; +x_106 = l_Lean_isEnumType___at___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___spec__2(x_104, x_2, x_3, x_4, x_5, x_6, x_7, x_73); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -if (lean_obj_tag(x_101) == 0) +if (lean_obj_tag(x_106) == 0) { -lean_object* x_102; lean_object* x_103; uint8_t x_104; -x_102 = lean_ctor_get(x_101, 0); -lean_inc(x_102); -x_103 = lean_ctor_get(x_102, 0); -lean_inc(x_103); -lean_dec(x_102); -x_104 = lean_unbox(x_103); -lean_dec(x_103); -if (x_104 == 0) +lean_object* x_107; lean_object* x_108; uint8_t x_109; +x_107 = lean_ctor_get(x_106, 0); +lean_inc(x_107); +x_108 = lean_ctor_get(x_107, 0); +lean_inc(x_108); +lean_dec(x_107); +x_109 = lean_unbox(x_108); +lean_dec(x_108); +if (x_109 == 0) { -lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; -x_105 = lean_ctor_get(x_101, 1); -lean_inc(x_105); -if (lean_is_exclusive(x_101)) { - lean_ctor_release(x_101, 0); - lean_ctor_release(x_101, 1); - x_106 = x_101; +lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; +x_110 = lean_ctor_get(x_106, 1); +lean_inc(x_110); +if (lean_is_exclusive(x_106)) { + lean_ctor_release(x_106, 0); + lean_ctor_release(x_106, 1); + x_111 = x_106; } else { - lean_dec_ref(x_101); - x_106 = lean_box(0); + lean_dec_ref(x_106); + x_111 = lean_box(0); } -x_107 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__4; -if (lean_is_scalar(x_106)) { - x_108 = lean_alloc_ctor(0, 2, 0); +x_112 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__5; +if (lean_is_scalar(x_111)) { + x_113 = lean_alloc_ctor(0, 2, 0); } else { - x_108 = x_106; + x_113 = x_111; } -lean_ctor_set(x_108, 0, x_107); -lean_ctor_set(x_108, 1, x_105); -return x_108; +lean_ctor_set(x_113, 0, x_112); +lean_ctor_set(x_113, 1, x_110); +return x_113; } else { -lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; -x_109 = lean_ctor_get(x_101, 1); -lean_inc(x_109); -if (lean_is_exclusive(x_101)) { - lean_ctor_release(x_101, 0); - lean_ctor_release(x_101, 1); - x_110 = x_101; +lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; +x_114 = lean_ctor_get(x_106, 1); +lean_inc(x_114); +if (lean_is_exclusive(x_106)) { + lean_ctor_release(x_106, 0); + lean_ctor_release(x_106, 1); + x_115 = x_106; } else { - lean_dec_ref(x_101); - x_110 = lean_box(0); + lean_dec_ref(x_106); + x_115 = lean_box(0); } -x_111 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__5; -if (lean_is_scalar(x_110)) { - x_112 = lean_alloc_ctor(0, 2, 0); +x_116 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__6; +if (lean_is_scalar(x_115)) { + x_117 = lean_alloc_ctor(0, 2, 0); } else { - x_112 = x_110; + x_117 = x_115; } -lean_ctor_set(x_112, 0, x_111); -lean_ctor_set(x_112, 1, x_109); -return x_112; +lean_ctor_set(x_117, 0, x_116); +lean_ctor_set(x_117, 1, x_114); +return x_117; } } else { -lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; -x_113 = lean_ctor_get(x_101, 0); -lean_inc(x_113); -x_114 = lean_ctor_get(x_101, 1); -lean_inc(x_114); -if (lean_is_exclusive(x_101)) { - lean_ctor_release(x_101, 0); - lean_ctor_release(x_101, 1); - x_115 = x_101; +lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; +x_118 = lean_ctor_get(x_106, 0); +lean_inc(x_118); +x_119 = lean_ctor_get(x_106, 1); +lean_inc(x_119); +if (lean_is_exclusive(x_106)) { + lean_ctor_release(x_106, 0); + lean_ctor_release(x_106, 1); + x_120 = x_106; } else { - lean_dec_ref(x_101); - x_115 = lean_box(0); + lean_dec_ref(x_106); + x_120 = lean_box(0); } -if (lean_is_scalar(x_115)) { - x_116 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_120)) { + x_121 = lean_alloc_ctor(1, 2, 0); } else { - x_116 = x_115; + x_121 = x_120; } -lean_ctor_set(x_116, 0, x_113); -lean_ctor_set(x_116, 1, x_114); -return x_116; +lean_ctor_set(x_121, 0, x_118); +lean_ctor_set(x_121, 1, x_119); +return x_121; } } else { -lean_object* x_117; lean_object* x_118; -lean_dec(x_99); +lean_object* x_122; lean_object* x_123; +lean_dec(x_104); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_117 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__6; -x_118 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_118, 0, x_117); -lean_ctor_set(x_118, 1, x_71); -return x_118; +x_122 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__7; +x_123 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_123, 0, x_122); +lean_ctor_set(x_123, 1, x_73); +return x_123; } } } else { -lean_object* x_119; lean_object* x_120; -lean_dec(x_72); +lean_object* x_124; lean_object* x_125; +lean_dec(x_74); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_119 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__7; -x_120 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_120, 0, x_119); -lean_ctor_set(x_120, 1, x_71); -return x_120; +x_124 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__8; +x_125 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_125, 0, x_124); +lean_ctor_set(x_125, 1, x_73); +return x_125; } } } @@ -7530,7 +7572,7 @@ static lean_object* _init_l___private_Lean_Server_Completion_0__Lean_Server_Comp lean_object* x_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_Completion_0__Lean_Server_Completion_truncate_go___closed__1; x_2 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_truncate_go___closed__2; -x_3 = lean_unsigned_to_nat(288u); +x_3 = lean_unsigned_to_nat(290u); x_4 = lean_unsigned_to_nat(25u); x_5 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_truncate_go___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -25133,7 +25175,7 @@ x_2 = lean_alloc_closure((void*)(l___private_Lean_Server_Completion_0__Lean_Serv return x_2; } } -static lean_object* _init_l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3___rarg___closed__1() { +static lean_object* _init_l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -25143,24 +25185,24 @@ x_3 = l_instInhabitedOfMonad___rarg(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3___rarg(lean_object* x_1) { +LEAN_EXPORT lean_object* l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3___rarg___closed__1; +x_2 = l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__1; x_3 = lean_panic_fn(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3(lean_object* x_1) { +LEAN_EXPORT lean_object* l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3___rarg), 1, 0); +x_2 = lean_alloc_closure((void*)(l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg), 1, 0); return x_2; } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__4___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { if (lean_obj_tag(x_4) == 0) @@ -25168,6 +25210,7 @@ if (lean_obj_tag(x_4) == 0) lean_object* x_6; lean_dec(x_3); lean_dec(x_2); +lean_dec(x_1); x_6 = l_List_reverse___rarg(x_5); return x_6; } @@ -25182,7 +25225,8 @@ x_8 = lean_ctor_get(x_4, 0); x_9 = lean_ctor_get(x_4, 1); lean_inc(x_3); lean_inc(x_2); -x_10 = l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg(x_1, x_2, x_3, x_8); +lean_inc(x_1); +x_10 = l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg(x_1, x_2, x_3, x_8); lean_ctor_set(x_4, 1, x_5); lean_ctor_set(x_4, 0, x_10); { @@ -25203,7 +25247,8 @@ lean_inc(x_12); lean_dec(x_4); lean_inc(x_3); lean_inc(x_2); -x_14 = l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg(x_1, x_2, x_3, x_12); +lean_inc(x_1); +x_14 = l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg(x_1, x_2, x_3, x_12); x_15 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_15, 0, x_14); lean_ctor_set(x_15, 1, x_5); @@ -25214,15 +25259,15 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__4(lean_object* x_1) { +LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_List_mapM_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__4___rarg___boxed), 5, 0); +x_2 = lean_alloc_closure((void*)(l_List_mapM_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3___rarg), 5, 0); return x_2; } } -static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__1() { +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__1() { _start: { lean_object* x_1; @@ -25230,7 +25275,7 @@ x_1 = lean_mk_string_unchecked("Lean.Server.InfoUtils", 21, 21); return x_1; } } -static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__2() { +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__2() { _start: { lean_object* x_1; @@ -25238,7 +25283,7 @@ x_1 = lean_mk_string_unchecked("Lean.Elab.InfoTree.visitM.go", 28, 28); return x_1; } } -static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__3() { +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__3() { _start: { lean_object* x_1; @@ -25246,20 +25291,20 @@ x_1 = lean_mk_string_unchecked("unexpected context-free info tree node", 38, 38) return x_1; } } -static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__4() { +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__1; -x_2 = l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__2; -x_3 = lean_unsigned_to_nat(56u); +x_1 = l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__1; +x_2 = l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__2; +x_3 = lean_unsigned_to_nat(62u); x_4 = lean_unsigned_to_nat(21u); -x_5 = l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__3; +x_5 = l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { if (lean_obj_tag(x_3) == 0) @@ -25283,8 +25328,9 @@ case 1: lean_object* x_9; lean_object* x_10; lean_dec(x_4); lean_dec(x_2); -x_9 = l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__4; -x_10 = l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3___rarg(x_9); +lean_dec(x_1); +x_9 = l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__4; +x_10 = l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg(x_9); return x_10; } default: @@ -25292,6 +25338,7 @@ return x_10; lean_object* x_11; lean_dec(x_4); lean_dec(x_2); +lean_dec(x_1); x_11 = lean_box(0); return x_11; } @@ -25319,92 +25366,117 @@ uint8_t x_16; x_16 = !lean_is_exclusive(x_3); if (x_16 == 0) { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; x_17 = lean_ctor_get(x_3, 0); x_18 = lean_ctor_get(x_4, 0); lean_inc(x_18); x_19 = lean_ctor_get(x_4, 1); lean_inc(x_19); lean_dec(x_4); +lean_inc(x_1); +lean_inc(x_19); +lean_inc(x_18); lean_inc(x_17); -x_20 = l_Lean_Elab_Info_updateContext_x3f(x_3, x_18); -x_21 = l_Lean_PersistentArray_toList___rarg(x_19); +x_20 = lean_apply_3(x_1, x_17, x_18, x_19); +x_21 = lean_unbox(x_20); +lean_dec(x_20); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; +lean_dec(x_1); x_22 = lean_box(0); +x_23 = lean_apply_4(x_2, x_17, x_18, x_19, x_22); +lean_ctor_set(x_3, 0, x_23); +return x_3; +} +else +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +lean_inc(x_17); +x_24 = l_Lean_Elab_Info_updateContext_x3f(x_3, x_18); +x_25 = l_Lean_PersistentArray_toList___rarg(x_19); +x_26 = lean_box(0); lean_inc(x_2); -x_23 = l_List_mapM_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__4___rarg(x_1, x_2, x_20, x_21, x_22); -x_24 = lean_apply_4(x_2, x_17, x_18, x_19, x_23); -x_25 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_25, 0, x_24); -return x_25; +x_27 = l_List_mapM_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3___rarg(x_1, x_2, x_24, x_25, x_26); +x_28 = lean_apply_4(x_2, x_17, x_18, x_19, x_27); +x_29 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_29, 0, x_28); +return x_29; +} } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_26 = lean_ctor_get(x_3, 0); -lean_inc(x_26); +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; +x_30 = lean_ctor_get(x_3, 0); +lean_inc(x_30); lean_dec(x_3); -x_27 = lean_ctor_get(x_4, 0); -lean_inc(x_27); -x_28 = lean_ctor_get(x_4, 1); -lean_inc(x_28); +x_31 = lean_ctor_get(x_4, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_4, 1); +lean_inc(x_32); lean_dec(x_4); -lean_inc(x_26); -x_29 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_29, 0, x_26); -x_30 = l_Lean_Elab_Info_updateContext_x3f(x_29, x_27); -x_31 = l_Lean_PersistentArray_toList___rarg(x_28); -x_32 = lean_box(0); +lean_inc(x_1); +lean_inc(x_32); +lean_inc(x_31); +lean_inc(x_30); +x_33 = lean_apply_3(x_1, x_30, x_31, x_32); +x_34 = lean_unbox(x_33); +lean_dec(x_33); +if (x_34 == 0) +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; +lean_dec(x_1); +x_35 = lean_box(0); +x_36 = lean_apply_4(x_2, x_30, x_31, x_32, x_35); +x_37 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_37, 0, x_36); +return x_37; +} +else +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; +lean_inc(x_30); +x_38 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_38, 0, x_30); +x_39 = l_Lean_Elab_Info_updateContext_x3f(x_38, x_31); +x_40 = l_Lean_PersistentArray_toList___rarg(x_32); +x_41 = lean_box(0); lean_inc(x_2); -x_33 = l_List_mapM_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__4___rarg(x_1, x_2, x_30, x_31, x_32); -x_34 = lean_apply_4(x_2, x_26, x_27, x_28, x_33); -x_35 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_35, 0, x_34); -return x_35; +x_42 = l_List_mapM_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3___rarg(x_1, x_2, x_39, x_40, x_41); +x_43 = lean_apply_4(x_2, x_30, x_31, x_32, x_42); +x_44 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_44, 0, x_43); +return x_44; +} } } default: { -lean_object* x_36; +lean_object* x_45; lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_36 = lean_box(0); -return x_36; -} -} -} -} +lean_dec(x_1); +x_45 = lean_box(0); +return x_45; } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___boxed), 4, 0); -return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; lean_object* x_5; -x_4 = lean_box(0); -x_5 = l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg(x_1, x_2, x_4, x_3); -return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___boxed), 3, 0); +x_2 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg), 4, 0); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_4; -x_4 = lean_box(0); +uint8_t x_4; +x_4 = 1; return x_4; } } @@ -25419,25 +25491,26 @@ return x_1; LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_4; lean_object* x_5; lean_object* x_6; +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_4 = lean_alloc_closure((void*)(l___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f_choose___rarg), 6, 2); lean_closure_set(x_4, 0, x_2); lean_closure_set(x_4, 1, x_3); -x_5 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___rarg___closed__1; -x_6 = l_Lean_Elab_InfoTree_visitM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg(x_5, x_4, x_1); -if (lean_obj_tag(x_6) == 0) +x_5 = lean_box(0); +x_6 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___rarg___closed__1; +x_7 = l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg(x_6, x_4, x_5, x_1); +if (lean_obj_tag(x_7) == 0) { -lean_object* x_7; -x_7 = lean_box(0); -return x_7; +lean_object* x_8; +x_8 = lean_box(0); +return x_8; } else { -lean_object* x_8; -x_8 = lean_ctor_get(x_6, 0); -lean_inc(x_8); -lean_dec(x_6); -return x_8; +lean_object* x_9; +x_9 = lean_ctor_get(x_7, 0); +lean_inc(x_9); +lean_dec(x_7); +return x_9; } } } @@ -25449,42 +25522,16 @@ x_2 = lean_alloc_closure((void*)(l___private_Lean_Server_Completion_0__Lean_Serv return x_2; } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__4___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; -x_6 = l_List_mapM_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__4___rarg(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_1); -return x_6; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -lean_object* x_5; -x_5 = l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg(x_1, x_2, x_3, x_4); -lean_dec(x_1); -return x_5; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l_Lean_Elab_InfoTree_visitM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg(x_1, x_2, x_3); -lean_dec(x_1); -return x_4; -} -} LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_4; +uint8_t x_4; lean_object* x_5; x_4 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___rarg___lambda__1(x_1, x_2, x_3); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -return x_4; +x_5 = lean_box(x_4); +return x_5; } } LEAN_EXPORT uint8_t l___private_Lean_Server_Completion_0__Lean_Server_Completion_findClosestInfoWithLocalContextAt_x3f_isBetter(lean_object* x_1, lean_object* x_2) { @@ -29447,7 +29494,7 @@ return x_53; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; uint8_t x_8; @@ -29729,24 +29776,24 @@ uint8_t x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_3 = lean_ctor_get_uint8(x_1, sizeof(void*)*1); x_4 = lean_ctor_get(x_1, 0); lean_inc(x_4); -x_5 = lean_array_get_size(x_4); -x_6 = lean_mk_empty_array_with_capacity(x_5); -x_7 = lean_unsigned_to_nat(0u); -x_8 = l_Array_mapIdxM_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts___spec__1(x_1, x_4, x_5, x_7, lean_box(0), x_6); -lean_dec(x_4); if (lean_is_exclusive(x_1)) { lean_ctor_release(x_1, 0); - x_9 = x_1; + x_5 = x_1; } else { lean_dec_ref(x_1); - x_9 = lean_box(0); + x_5 = lean_box(0); } -x_10 = lean_array_get_size(x_8); +x_6 = lean_array_get_size(x_4); +x_7 = lean_mk_empty_array_with_capacity(x_6); +x_8 = lean_unsigned_to_nat(0u); +x_9 = l_Array_mapFinIdxM_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts___spec__1(x_4, x_4, x_6, x_8, lean_box(0), x_7); +lean_dec(x_4); +x_10 = lean_array_get_size(x_9); x_11 = lean_unsigned_to_nat(1u); x_12 = lean_nat_sub(x_10, x_11); x_13 = lean_nat_dec_lt(x_12, x_10); lean_dec(x_10); -x_14 = lean_array_size(x_8); +x_14 = lean_array_size(x_9); x_15 = 0; if (x_13 == 0) { @@ -29778,7 +29825,7 @@ goto block_20; else { lean_object* x_27; lean_object* x_28; -x_27 = lean_array_fget(x_8, x_12); +x_27 = lean_array_fget(x_9, x_12); lean_dec(x_12); x_28 = lean_ctor_get(x_27, 5); lean_inc(x_28); @@ -29806,12 +29853,12 @@ goto block_20; lean_object* x_17; lean_object* x_18; lean_object* x_19; x_17 = lean_string_length(x_16); lean_dec(x_16); -x_18 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts___spec__2(x_17, x_14, x_15, x_8); +x_18 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts___spec__2(x_17, x_14, x_15, x_9); lean_dec(x_17); -if (lean_is_scalar(x_9)) { +if (lean_is_scalar(x_5)) { x_19 = lean_alloc_ctor(0, 1, 1); } else { - x_19 = x_9; + x_19 = x_5; } lean_ctor_set(x_19, 0, x_18); lean_ctor_set_uint8(x_19, sizeof(void*)*1, x_3); @@ -29840,11 +29887,11 @@ return x_1; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; -x_7 = l_Array_mapIdxM_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts___spec__1(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Array_mapFinIdxM_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts___spec__1(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_2); lean_dec(x_1); return x_7; @@ -30882,6 +30929,8 @@ l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindFo lean_mark_persistent(l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__6); l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__7 = _init_l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__7(); lean_mark_persistent(l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__7); +l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__8 = _init_l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__8(); +lean_mark_persistent(l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__8); l___private_Lean_Server_Completion_0__Lean_Server_Completion_addKeywordCompletionItem___closed__1 = _init_l___private_Lean_Server_Completion_0__Lean_Server_Completion_addKeywordCompletionItem___closed__1(); lean_mark_persistent(l___private_Lean_Server_Completion_0__Lean_Server_Completion_addKeywordCompletionItem___closed__1); l___private_Lean_Server_Completion_0__Lean_Server_Completion_addKeywordCompletionItem___closed__2 = _init_l___private_Lean_Server_Completion_0__Lean_Server_Completion_addKeywordCompletionItem___closed__2(); @@ -30976,16 +31025,16 @@ l___private_Lean_Server_Completion_0__Lean_Server_Completion_optionCompletion___ lean_mark_persistent(l___private_Lean_Server_Completion_0__Lean_Server_Completion_optionCompletion___closed__6); l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_tacticCompletion___spec__1___boxed__const__1 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_tacticCompletion___spec__1___boxed__const__1(); lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_tacticCompletion___spec__1___boxed__const__1); -l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3___rarg___closed__1 = _init_l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3___rarg___closed__1(); -lean_mark_persistent(l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3___rarg___closed__1); -l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__1 = _init_l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__1(); -lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__1); -l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__2 = _init_l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__2(); -lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__2); -l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__3 = _init_l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__3(); -lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__3); -l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__4 = _init_l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__4(); -lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__4); +l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__1 = _init_l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__1(); +lean_mark_persistent(l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__1); +l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__1 = _init_l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__1(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__1); +l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__2 = _init_l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__2(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__2); +l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__3 = _init_l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__3(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__3); +l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__4 = _init_l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__4(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__4); l___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___rarg___closed__1 = _init_l___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___rarg___closed__1(); lean_mark_persistent(l___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___rarg___closed__1); l___private_Lean_Server_Completion_0__Lean_Server_Completion_findClosestInfoWithLocalContextAt_x3f___closed__1 = _init_l___private_Lean_Server_Completion_0__Lean_Server_Completion_findClosestInfoWithLocalContextAt_x3f___closed__1(); diff --git a/stage0/stdlib/Lean/Server/CompletionItemData.c b/stage0/stdlib/Lean/Server/CompletionItemData.c index 0ee0daac90c9..76668c813afe 100644 --- a/stage0/stdlib/Lean/Server/CompletionItemData.c +++ b/stage0/stdlib/Lean/Server/CompletionItemData.c @@ -23,6 +23,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Server_CompletionItemData_0__Lean_Lsp_ static lean_object* l___private_Lean_Server_CompletionItemData_0__Lean_Lsp_fromJsonCompletionItemData____x40_Lean_Server_CompletionItemData___hyg_15____closed__12; static lean_object* l___private_Lean_Server_CompletionItemData_0__Lean_Lsp_fromJsonCompletionItemData____x40_Lean_Server_CompletionItemData___hyg_15____closed__10; static lean_object* l___private_Lean_Server_CompletionItemData_0__Lean_Lsp_fromJsonCompletionItemData____x40_Lean_Server_CompletionItemData___hyg_15____closed__13; +lean_object* l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Lsp_CompletionItem_getFileSource_x21___closed__2; LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Server_CompletionItemData_0__Lean_Lsp_fromJsonCompletionItemData____x40_Lean_Server_CompletionItemData___hyg_15____spec__1(lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); @@ -40,7 +41,6 @@ lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2476_(lean_object*); static lean_object* l___private_Lean_Server_CompletionItemData_0__Lean_Lsp_fromJsonCompletionItemData____x40_Lean_Server_CompletionItemData___hyg_15____closed__5; -lean_object* l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_CompletionItemData_0__Lean_Lsp_toJsonCompletionItemData____x40_Lean_Server_CompletionItemData___hyg_82_(lean_object*); static lean_object* l_Lean_Lsp_CompletionItem_getFileSource_x21___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Server_CompletionItemData_0__Lean_Lsp_fromJsonCompletionItemData____x40_Lean_Server_CompletionItemData___hyg_15_(lean_object*); @@ -321,7 +321,7 @@ x_7 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_7, 0, x_6); lean_ctor_set(x_7, 1, x_5); x_8 = l___private_Lean_Server_CompletionItemData_0__Lean_Lsp_toJsonCompletionItemData____x40_Lean_Server_CompletionItemData___hyg_82____closed__1; -x_9 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } diff --git a/stage0/stdlib/Lean/Server/FileWorker/RequestHandling.c b/stage0/stdlib/Lean/Server/FileWorker/RequestHandling.c index a36ad45017a6..552945b4b3aa 100644 --- a/stage0/stdlib/Lean/Server/FileWorker/RequestHandling.c +++ b/stage0/stdlib/Lean/Server/FileWorker/RequestHandling.c @@ -403,6 +403,7 @@ LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileW LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentHighlight_highlightReturn_x3f___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getTrailingSize(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12731____spec__7___lambda__1(lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_levelZero; @@ -493,7 +494,6 @@ LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleSemanticTokens___lambda_ LEAN_EXPORT uint8_t l_Lean_Server_FileWorker_handleHover___lambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12731_(lean_object*); static lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__8___closed__11; -lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12731____spec__37___lambda__1(lean_object*); static lean_object* l___private_Lean_Server_FileWorker_RequestHandling_0__Lean_Server_FileWorker_fromJsonAbsoluteLspSemanticToken____x40_Lean_Server_FileWorker_RequestHandling___hyg_8744____closed__11; static lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12731____spec__2___closed__1; @@ -19925,7 +19925,7 @@ x_20 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_20, 0, x_7); lean_ctor_set(x_20, 1, x_19); x_21 = l_Lean_Server_FileWorker_handleCompletion___lambda__1___closed__1; -x_22 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_20, x_21); +x_22 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_20, x_21); x_23 = l_Lean_Json_mkObj(x_22); return x_23; } diff --git a/stage0/stdlib/Lean/Server/FileWorker/WidgetRequests.c b/stage0/stdlib/Lean/Server/FileWorker/WidgetRequests.c index c37c057dd348..128d1eb8ff7d 100644 --- a/stage0/stdlib/Lean/Server/FileWorker/WidgetRequests.c +++ b/stage0/stdlib/Lean/Server/FileWorker/WidgetRequests.c @@ -154,6 +154,7 @@ lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1387____spec__2___closed__1; static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1387____closed__2; LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1387____spec__1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); extern lean_object* l_Lean_Lsp_instFromJsonLocationLink; static lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_520____closed__6; extern lean_object* l_Lean_Widget_instRpcEncodableInteractiveTermGoal; @@ -179,7 +180,6 @@ LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodableInfoPopup_enc____x40_Lean static lean_object* l_Lean_Widget_instRpcEncodableGetGoToLocationParams___closed__2; static lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_58____closed__33; lean_object* l_Lean_Server_instRpcEncodableWithRpcRefOfTypeName_rpcEncode___rarg(lean_object*, lean_object*, lean_object*); -lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1450____spec__1___closed__1; static lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_58____closed__26; static lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_58____closed__12; @@ -769,7 +769,7 @@ x_12 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_12, 0, x_7); lean_ctor_set(x_12, 1, x_11); x_13 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodablePacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_204____closed__1; -x_14 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); +x_14 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); x_15 = l_Lean_Json_mkObj(x_14); return x_15; } @@ -803,7 +803,7 @@ x_26 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_26, 0, x_21); lean_ctor_set(x_26, 1, x_25); x_27 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodablePacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_204____closed__1; -x_28 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_26, x_27); +x_28 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_26, x_27); x_29 = l_Lean_Json_mkObj(x_28); return x_29; } @@ -1710,7 +1710,7 @@ x_17 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_17, 0, x_8); lean_ctor_set(x_17, 1, x_16); x_18 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodablePacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_204____closed__1; -x_19 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_17, x_18); +x_19 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_17, x_18); x_20 = l_Lean_Json_mkObj(x_19); return x_20; } @@ -4338,7 +4338,7 @@ x_5 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_5, 0, x_3); lean_ctor_set(x_5, 1, x_4); x_6 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodablePacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_204____closed__1; -x_7 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_5, x_6); +x_7 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_5, x_6); x_8 = l_Lean_Json_mkObj(x_7); return x_8; } @@ -4573,7 +4573,7 @@ x_12 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_12, 0, x_7); lean_ctor_set(x_12, 1, x_11); x_13 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodablePacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_204____closed__1; -x_14 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); +x_14 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); x_15 = l_Lean_Json_mkObj(x_14); return x_15; } @@ -4607,7 +4607,7 @@ x_26 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_26, 0, x_21); lean_ctor_set(x_26, 1, x_25); x_27 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodablePacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_204____closed__1; -x_28 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_26, x_27); +x_28 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_26, x_27); x_29 = l_Lean_Json_mkObj(x_28); return x_29; } diff --git a/stage0/stdlib/Lean/Server/InfoUtils.c b/stage0/stdlib/Lean/Server/InfoUtils.c index 5977b9022882..01e0c6c57405 100644 --- a/stage0/stdlib/Lean/Server/InfoUtils.c +++ b/stage0/stdlib/Lean/Server/InfoUtils.c @@ -15,36 +15,31 @@ extern "C" { #endif LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*); -LEAN_EXPORT lean_object* l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__19___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__6___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* l_Lean_Meta_ppExpr(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterMapTR_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__1___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_goalsAt_x3f(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t); -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_fmtHover_x3f_fmtModule_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_InfoTree_goalsAt_x3f_isEmptyBy(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__11___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___lambda__1___boxed(lean_object*); -LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__7(lean_object*); static lean_object* l_Lean_Elab_InfoTree_visitM_go___rarg___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__21___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* l_Lean_PrettyPrinter_ppSignature(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_hasSorry_go___spec__16___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_getConstInfo___at_Lean_Meta_mkConstWithFreshMVarLevels___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_InfoTree_visitM_go___rarg___closed__3; +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_visitM_x27___spec__3(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlFromMAux___at_Lean_Elab_InfoTree_foldInfo_go___spec__15(lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_visitM_go___spec__1___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__24___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); size_t lean_usize_shift_right(size_t, size_t); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__39___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__19(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_foldlM___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__17(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_smallestInfo_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__21___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__17___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__12; LEAN_EXPORT lean_object* l_Lean_Elab_Info_isTerm___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_occursInside_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_docString_x3f___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -56,29 +51,27 @@ LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_InfoTree_ uint8_t l_List_all___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Info_fmtHover_x3f_fmtModule_x3f___closed__5; LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__5___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__12___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__26___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_visitM_x27___spec__2___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___closed__1; +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__28___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_goalsAt_x3f___spec__8___boxed(lean_object*, lean_object*); uint8_t l_Lean_Exception_isInterrupt(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__38___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9; -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__3___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__16(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlFromMAux___at_Lean_Elab_InfoTree_foldInfo_go___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_foldlM___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__14___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_FileMap_toPosition(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__49(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_foldInfo_go(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_getCompletionInfos(lean_object*); static lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__7___closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_smallestInfo_x3f___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__7___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__2(lean_object*); @@ -89,18 +82,17 @@ LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic___lamb lean_object* l_Lean_findDocString_x3f(lean_object*, lean_object*, uint8_t, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isApp(lean_object*); -LEAN_EXPORT lean_object* l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__13___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_toString(lean_object*, uint8_t, lean_object*); +LEAN_EXPORT uint8_t l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__12(lean_object*, lean_object*, lean_object*); static lean_object* l_List_mapTR_loop___at_Lean_Elab_InfoTree_smallestInfo_x3f___spec__1___closed__4; +LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__16(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__53(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_foldInfo_go___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__12___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_foldlM___at_Lean_Elab_InfoTree_foldInfo_go___spec__14___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_InfoTree_hasSorry_go___spec__37(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__17(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlMAux___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -123,11 +115,14 @@ LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_goalsAt_x3f_h LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__22___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getTailPos_x3f(lean_object*, uint8_t); static lean_object* l_Lean_Elab_InfoTree_visitM_go___rarg___closed__2; +LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_InfoTree_hasSorry_go___spec__17(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_visitM_x27___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__22___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_List_mapTR_loop___at_Lean_Elab_InfoTree_smallestInfo_x3f___spec__1___closed__3; static lean_object* l_Lean_Elab_Info_fmtHover_x3f_fmtTermAndModule_x3f___lambda__1___closed__5; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__22(lean_object*); +LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__14(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_InfoTree_hasSorry_go___spec__27___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_deepestNodes(lean_object*); @@ -143,7 +138,7 @@ extern lean_object* l_Lean_LocalContext_empty; LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_hasSorry_go___spec__11(lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__26___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__17___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__13___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__7___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_hasSorry_go___spec__41(lean_object*, lean_object*, lean_object*); @@ -151,6 +146,7 @@ LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_InfoTree_ lean_object* l_Lean_instInhabitedPersistentArrayNode(lean_object*); lean_object* l_Lean_PersistentArray_toList___rarg(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__30(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_visitM_x27___spec__3___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__8___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlMAux___at_Lean_Elab_InfoTree_foldInfo_go___spec__23___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_docString_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -160,7 +156,6 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldI LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_occursInOrOnBoundary___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__9(lean_object*); -LEAN_EXPORT uint8_t l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__18(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlFromMAux___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__15(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_goalsAt_x3f___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_docString_x3f___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -170,6 +165,7 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldI lean_object* l_Lean_Elab_CompletionInfo_stx(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__11(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__5(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_smallestInfo_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_hasSorry_go___spec__46(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_hasSorry_go___spec__1___boxed(lean_object*, lean_object*, lean_object*); @@ -179,19 +175,17 @@ LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_goalsAt_ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__18___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__4___closed__2; LEAN_EXPORT uint8_t l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4(lean_object*); LEAN_EXPORT uint8_t l_Lean_PersistentArray_anyMAux___at_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Info_fmtHover_x3f_fmtTermAndModule_x3f___lambda__1___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_visitM_x27___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__3(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__4___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27(lean_object*); -LEAN_EXPORT lean_object* l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__16___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlMAux___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__16___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__4(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_fmtHover_x3f_isAtomicFormat___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_fmtHover_x3f___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__21(lean_object*); -static lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__19___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__19___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_fmtHover_x3f(lean_object*, lean_object*, lean_object*); @@ -205,6 +199,7 @@ size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__9(lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__7___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_deepestNodes___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_InfoTree_hasSorry_go___spec__52(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__11(lean_object*); LEAN_EXPORT lean_object* l_List_max_x3f___at_Lean_Elab_InfoTree_goalsAt_x3f___spec__7(lean_object*); @@ -231,6 +226,7 @@ LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_goa LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlMAux___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__23___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Info_docString_x3f___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_PersistentArray_foldlM___at_Lean_Elab_InfoTree_foldInfo_go___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Info_fmtHover_x3f_fmtTermAndModule_x3f___lambda__1___closed__8; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__21___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_goalsAt_x3f___spec__8(lean_object*, lean_object*); @@ -238,16 +234,15 @@ static lean_object* l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___lambda__2 LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__25(lean_object*); LEAN_EXPORT lean_object* l_List_filterMapTR_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__7(lean_object*); +LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_visitM_x27___spec__2(lean_object*); LEAN_EXPORT uint8_t l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__10(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT uint8_t l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__13(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__13(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__14(lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__5(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_range_x3f___boxed(lean_object*); LEAN_EXPORT lean_object* l_List_filterTR_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__4(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlMAux___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__23___rarg(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Info_updateContext_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__1___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_bindTR_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__2___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_visitM_go___spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_hasSorry_go___spec__11___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_type_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -267,17 +262,17 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldI lean_object* l_Lean_Elab_PartialContextInfo_mergeIntoOuter_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__13(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__18___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__17___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__20(lean_object*); +LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___lambda__1___boxed(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__30___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getKind(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_isSmaller___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_goalsAt_x3f___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_CompletionInfo_lctx(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlMAux___at_Lean_Elab_InfoTree_foldInfo_go___spec__10(lean_object*); -LEAN_EXPORT lean_object* l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__11___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__54(lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5___rarg(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__7___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__23(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_InfoTree_hasSorry_go___spec__17___boxed(lean_object*, lean_object*, lean_object*); @@ -317,6 +312,7 @@ static lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArra LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_InfoTree_hasSorry_go___spec__42___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__8___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__6(lean_object*); +static lean_object* l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlFromMAux___at_Lean_Elab_InfoTree_foldInfo_go___spec__15___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Elab_InfoTree_getCompletionInfos___closed__1; LEAN_EXPORT lean_object* l_Array_getMax_x3f___at_Lean_Elab_InfoTree_smallestInfo_x3f___spec__2(lean_object*); @@ -326,7 +322,7 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldI lean_object* l_Lean_Expr_constName_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_InfoTree_hasSorry_go___spec__22(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__19(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_mapTR_loop___at_Lean_Elab_InfoTree_smallestInfo_x3f___spec__1___closed__1; static lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__4___closed__6; LEAN_EXPORT lean_object* l_Lean_PersistentArray_foldlM___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__14(lean_object*); @@ -334,13 +330,14 @@ static lean_object* l_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic___closed__2 LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_hasSorry_go___spec__26___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__18___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__48(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlMAux___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__16(lean_object*); static lean_object* l_Lean_Elab_Info_fmtHover_x3f_fmtModule_x3f___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_visitM_x27___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__4(lean_object*); uint8_t lean_name_eq(lean_object*, lean_object*); -static lean_object* l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5___rarg___closed__1; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__24(lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__7___closed__1; @@ -352,8 +349,8 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldI LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__17___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_fmtHover_x3f___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Info_fmtHover_x3f_fmtTermAndModule_x3f___lambda__1___closed__6; +LEAN_EXPORT lean_object* l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__15___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___lambda__1(lean_object*); lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__50___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__50(lean_object*, lean_object*, size_t, size_t, lean_object*); @@ -369,45 +366,50 @@ uint8_t l_Lean_Syntax_isIdent(lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__19___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_InfoTree_smallestInfo_x3f___spec__1(lean_object*, lean_object*); -LEAN_EXPORT uint8_t l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__11(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8; +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__3(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__21(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlMAux___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__23(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__18___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_goalsAt_x3f___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlMAux___at_Lean_Elab_InfoTree_foldInfo_go___spec__10___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_hasSorry_go___spec__51(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__11; +LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__19___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__7___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__4___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlMAux___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__3(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_visitM_x27___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_usize_to_nat(size_t); LEAN_EXPORT lean_object* l_Lean_Elab_Info_pos_x3f___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_docString_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__33___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__6(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_collectNodesBottomUp(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__35___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_instantiateMVars___at___private_Lean_Meta_Basic_0__Lean_Meta_isClassApp_x3f___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___lambda__2(lean_object*); +LEAN_EXPORT lean_object* l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__43___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__4___closed__3; +LEAN_EXPORT lean_object* l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__18(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_userName(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlMAux___at_Lean_Elab_InfoTree_foldInfo_go___spec__23(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__13___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_fmtHover_x3f_fmtTermAndModule_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_foldlM___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__14___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__40(lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5(lean_object*); lean_object* l_panic___at_Lean_Parser_ParserState_mkUnexpectedTokenErrors___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_smallestInfo_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___closed__2; +static lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Info_docString_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_InfoTree_hasSorry_go___spec__47(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__18___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__33(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__24___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__17___boxed(lean_object*, lean_object*); uint8_t l_Lean_Syntax_isToken(lean_object*, lean_object*); uint8_t l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_365____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__22___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -415,7 +417,6 @@ LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry uint8_t l_Lean_Name_hasMacroScopes(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlMAux___at_Lean_Elab_InfoTree_foldInfo_go___spec__3___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__26___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_visitM_x27___spec__1(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlMAux___at_Lean_Elab_InfoTree_foldInfo_go___spec__16___rarg(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_lexOrd___elambda__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_termGoalAt_x3f(lean_object*, lean_object*); @@ -423,10 +424,12 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldI uint8_t l_String_Range_contains(lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__44(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_visitM_x27___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_InfoTree_visitM_go___rarg___closed__4; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__28(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_hasSorry_go___spec__6(lean_object*, lean_object*, lean_object*); +static lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___closed__2; LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_hasSorry_go___spec__26(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__8(lean_object*, lean_object*, size_t, size_t, lean_object*); @@ -435,7 +438,6 @@ static lean_object* l_Lean_Elab_Info_fmtHover_x3f_fmtModule_x3f___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__19___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlMAux___at_Lean_Elab_InfoTree_foldInfo_go___spec__10___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_visitM_go___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_bindTR_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__35(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_deepestNodes___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_fmtHover_x3f___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -447,8 +449,8 @@ lean_object* l_Lean_instantiateMVars___at___private_Lean_Meta_Basic_0__Lean_Meta LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__38(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__34___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_goalsAt_x3f_isEmptyBy___boxed(lean_object*); -LEAN_EXPORT lean_object* l_List_bindTR_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlMAux___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__10___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__17(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__9___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__43(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_fmtHover_x3f___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -463,14 +465,16 @@ LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_Persisten LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__18___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlMAux___at_Lean_Elab_InfoTree_foldInfo_go___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___lambda__2(lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__3(lean_object*); +LEAN_EXPORT lean_object* l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__15(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__11___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__6___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_Format_joinSep___at_Prod_repr___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_InfoTree_hasSorry_go___spec__7(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__6(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlFromMAux___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__15___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__6(lean_object*); uint8_t l_instDecidableRelLe___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__12___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_hasSorry_go___spec__46___boxed(lean_object*, lean_object*, lean_object*); @@ -482,12 +486,12 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldI LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__25(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_goalsAt_x3f___lambda__1___boxed(lean_object*); lean_object* lean_panic_fn(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__19(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_int_dec_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_fmtHover_x3f_fmtTermAndModule_x3f___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__12___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__20___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_getCompletionInfos___lambda__1(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__6___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__24(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_hasSorry_go___spec__36___boxed(lean_object*, lean_object*, lean_object*); @@ -500,22 +504,19 @@ lean_object* l_Lean_Elab_TermInfo_runMetaM___rarg(lean_object*, lean_object*, le LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_hasSorry_go___spec__6___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__55(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_InfoTree_hasSorry_go___spec__2(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__3___rarg___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_range_x3f(lean_object*); static lean_object* l_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__14(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_deepestNodes___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlFromMAux___at_Lean_Elab_InfoTree_foldInfo_go___spec__2___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* l_List_foldl___at_Array_appendList___spec__1___rarg(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_Info_fmtHover_x3f_fmtModule_x3f___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__7(lean_object*, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__6(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__13___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* l_Lean_Environment_getModuleIdxFor_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__18(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_visitM_x27___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_reverse___rarg(lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_InfoTree_goalsAt_x3f___spec__6(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_visitM_go___spec__1(lean_object*, lean_object*); @@ -527,7 +528,7 @@ uint8_t l_Lean_Syntax_structEq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_foldlM___at_Lean_Elab_InfoTree_foldInfo_go___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_InfoTree_goalsAt_x3f___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_hasSorry_go___spec__21___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterTR_loop___at_Lean_Elab_InfoTree_goalsAt_x3f___spec__9___boxed(lean_object*, lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); @@ -550,7 +551,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Info_lctx(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__25___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_getMax_x3f___at_Lean_Elab_InfoTree_smallestInfo_x3f___spec__2___boxed(lean_object*); -LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__15(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__20___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_goalsAt_x3f___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -564,9 +564,10 @@ size_t lean_usize_shift_left(size_t, size_t); lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_int_dec_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__39(lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___lambda__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_foldInfoTree___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Info_fmtHover_x3f_fmtTermAndModule_x3f___lambda__1___closed__3; +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__2___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_InfoTree_hasSorry_go___spec__22___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__18(lean_object*, lean_object*, size_t, size_t, lean_object*); @@ -585,12 +586,12 @@ LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry lean_object* l_Lean_RBNode_find___at_Lean_NameMap_find_x3f___spec__1___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__7(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__12(lean_object*); -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlFromMAux___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__2___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Elab_Info_fmtHover_x3f_fmtTermAndModule_x3f___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__24(lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_goalsAt_x3f___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t); static lean_object* l_Lean_Elab_Info_fmtHover_x3f_fmtTermAndModule_x3f___lambda__1___closed__4; +LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___lambda__2___boxed(lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_InfoTree_hasSorry_go___spec__42(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f(lean_object*, lean_object*, uint8_t, uint8_t, uint8_t); @@ -621,10 +622,8 @@ uint8_t l_Lean_Expr_isSyntheticSorry(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_hasSorry_go___spec__1(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalContext_findFVar_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__6___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__25___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_fmtHover_x3f_fmtTermAndModule_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___lambda__2___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_stx___boxed(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__26___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__34(lean_object*, lean_object*, size_t, size_t, lean_object*); @@ -632,7 +631,6 @@ LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_hasSorry_go___spec__36(lean_object*, lean_object*, lean_object*); size_t lean_usize_land(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_foldInfo(lean_object*); -LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__20(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__5(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_fmtHover_x3f_fmtTermAndModule_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_Info_contains(lean_object*, lean_object*, uint8_t); @@ -750,29 +748,43 @@ x_10 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_8, x_9); return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, uint8_t x_8) { _start: { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +if (x_8 == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +lean_dec(x_7); +x_9 = lean_box(0); +x_10 = lean_apply_4(x_1, x_2, x_3, x_4, x_9); +x_11 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_go___rarg___lambda__1), 2, 1); +lean_closure_set(x_11, 0, x_5); +x_12 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_10, x_11); +return x_12; +} +else +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +lean_inc(x_2); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_2); +x_14 = l_Lean_Elab_Info_updateContext_x3f(x_13, x_3); +x_15 = l_Lean_PersistentArray_toList___rarg(x_4); +x_16 = lean_box(0); lean_inc(x_1); -x_9 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_9, 0, x_1); -x_10 = l_Lean_Elab_Info_updateContext_x3f(x_9, x_2); -x_11 = l_Lean_PersistentArray_toList___rarg(x_3); -x_12 = lean_box(0); +lean_inc(x_5); +x_17 = l_List_mapM_loop___at_Lean_Elab_InfoTree_visitM_go___spec__2___rarg(x_5, x_7, x_1, x_14, x_15, x_16); lean_inc(x_6); -lean_inc(x_4); -x_13 = l_List_mapM_loop___at_Lean_Elab_InfoTree_visitM_go___spec__2___rarg(x_4, x_5, x_6, x_10, x_11, x_12); -lean_inc(x_7); -x_14 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_go___rarg___lambda__2), 7, 6); -lean_closure_set(x_14, 0, x_6); -lean_closure_set(x_14, 1, x_1); -lean_closure_set(x_14, 2, x_2); -lean_closure_set(x_14, 3, x_3); -lean_closure_set(x_14, 4, x_4); -lean_closure_set(x_14, 5, x_7); -x_15 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_13, x_14); -return x_15; +x_18 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_go___rarg___lambda__2), 7, 6); +lean_closure_set(x_18, 0, x_1); +lean_closure_set(x_18, 1, x_2); +lean_closure_set(x_18, 2, x_3); +lean_closure_set(x_18, 3, x_4); +lean_closure_set(x_18, 4, x_5); +lean_closure_set(x_18, 5, x_6); +x_19 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_17, x_18); +return x_19; +} } } static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___rarg___closed__1() { @@ -805,7 +817,7 @@ static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___rarg___closed__4() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Elab_InfoTree_visitM_go___rarg___closed__1; x_2 = l_Lean_Elab_InfoTree_visitM_go___rarg___closed__2; -x_3 = lean_unsigned_to_nat(56u); +x_3 = lean_unsigned_to_nat(62u); x_4 = lean_unsigned_to_nat(21u); x_5 = l_Lean_Elab_InfoTree_visitM_go___rarg___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -895,13 +907,13 @@ lean_inc(x_20); x_24 = lean_apply_3(x_2, x_20, x_21, x_22); lean_inc(x_23); x_25 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_go___rarg___lambda__3___boxed), 8, 7); -lean_closure_set(x_25, 0, x_20); -lean_closure_set(x_25, 1, x_21); -lean_closure_set(x_25, 2, x_22); -lean_closure_set(x_25, 3, x_1); -lean_closure_set(x_25, 4, x_2); -lean_closure_set(x_25, 5, x_3); -lean_closure_set(x_25, 6, x_23); +lean_closure_set(x_25, 0, x_3); +lean_closure_set(x_25, 1, x_20); +lean_closure_set(x_25, 2, x_21); +lean_closure_set(x_25, 3, x_22); +lean_closure_set(x_25, 4, x_1); +lean_closure_set(x_25, 5, x_23); +lean_closure_set(x_25, 6, x_2); x_26 = lean_apply_4(x_23, lean_box(0), lean_box(0), x_24, x_25); return x_26; } @@ -937,18 +949,18 @@ return x_3; LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___rarg___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_9; -x_9 = l_Lean_Elab_InfoTree_visitM_go___rarg___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +uint8_t x_9; lean_object* x_10; +x_9 = lean_unbox(x_8); lean_dec(x_8); -return x_9; +x_10 = l_Lean_Elab_InfoTree_visitM_go___rarg___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_9); +return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_5; lean_object* x_6; -x_5 = lean_box(0); -x_6 = l_Lean_Elab_InfoTree_visitM_go___rarg(x_1, x_2, x_3, x_5, x_4); +lean_object* x_6; +x_6 = l_Lean_Elab_InfoTree_visitM_go___rarg(x_1, x_2, x_3, x_4, x_5); return x_6; } } @@ -956,24 +968,251 @@ LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM(lean_object* x_1, lean_obje _start: { lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM___rarg), 4, 0); +x_3 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM___rarg), 5, 0); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_visitM_x27___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_visitM_x27___spec__2___rarg(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_5; lean_object* x_6; -x_5 = lean_box(0); -x_6 = l_Lean_Elab_InfoTree_visitM_go___rarg(x_1, x_2, x_3, x_5, x_4); -return x_6; +lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_3 = lean_box(0); +x_4 = l_instInhabitedOfMonad___rarg(x_1, x_3); +x_5 = lean_panic_fn(x_4, x_2); +return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_visitM_x27___spec__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_visitM_x27___spec__2(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_visitM_x27___spec__1___rarg), 4, 0); +x_2 = lean_alloc_closure((void*)(l_panic___at_Lean_Elab_InfoTree_visitM_x27___spec__2___rarg), 2, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_visitM_x27___spec__3___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; lean_object* x_9; +x_8 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_8, 0, x_7); +lean_ctor_set(x_8, 1, x_1); +x_9 = l_List_mapM_loop___at_Lean_Elab_InfoTree_visitM_x27___spec__3___rarg(x_2, x_3, x_4, x_5, x_6, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_visitM_x27___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = l_List_reverse___rarg(x_6); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_11 = lean_ctor_get(x_5, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_5, 1); +lean_inc(x_12); +lean_dec(x_5); +x_13 = lean_ctor_get(x_1, 1); +lean_inc(x_13); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_visitM_x27___spec__1___rarg(x_1, x_2, x_3, x_4, x_11); +x_15 = lean_alloc_closure((void*)(l_List_mapM_loop___at_Lean_Elab_InfoTree_visitM_x27___spec__3___rarg___lambda__1), 7, 6); +lean_closure_set(x_15, 0, x_6); +lean_closure_set(x_15, 1, x_1); +lean_closure_set(x_15, 2, x_2); +lean_closure_set(x_15, 3, x_3); +lean_closure_set(x_15, 4, x_4); +lean_closure_set(x_15, 5, x_12); +x_16 = lean_apply_4(x_13, lean_box(0), lean_box(0), x_14, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_visitM_x27___spec__3(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_List_mapM_loop___at_Lean_Elab_InfoTree_visitM_x27___spec__3___rarg), 6, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_visitM_x27___spec__1___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, uint8_t x_8) { +_start: +{ +if (x_8 == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +lean_dec(x_7); +x_9 = lean_box(0); +x_10 = lean_apply_4(x_1, x_2, x_3, x_4, x_9); +x_11 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_go___rarg___lambda__1), 2, 1); +lean_closure_set(x_11, 0, x_5); +x_12 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_10, x_11); +return x_12; +} +else +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +lean_inc(x_2); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_2); +x_14 = l_Lean_Elab_Info_updateContext_x3f(x_13, x_3); +x_15 = l_Lean_PersistentArray_toList___rarg(x_4); +x_16 = lean_box(0); +lean_inc(x_1); +lean_inc(x_5); +x_17 = l_List_mapM_loop___at_Lean_Elab_InfoTree_visitM_x27___spec__3___rarg(x_5, x_7, x_1, x_14, x_15, x_16); +lean_inc(x_6); +x_18 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_go___rarg___lambda__2), 7, 6); +lean_closure_set(x_18, 0, x_1); +lean_closure_set(x_18, 1, x_2); +lean_closure_set(x_18, 2, x_3); +lean_closure_set(x_18, 3, x_4); +lean_closure_set(x_18, 4, x_5); +lean_closure_set(x_18, 5, x_6); +x_19 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_17, x_18); +return x_19; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_visitM_x27___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_4) == 0) +{ +switch (lean_obj_tag(x_5)) { +case 0: +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_6 = lean_ctor_get(x_5, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_5, 1); +lean_inc(x_7); +lean_dec(x_5); +x_8 = l_Lean_Elab_PartialContextInfo_mergeIntoOuter_x3f(x_6, x_4); +x_4 = x_8; +x_5 = x_7; +goto _start; +} +case 1: +{ +lean_object* x_10; lean_object* x_11; +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +x_10 = l_Lean_Elab_InfoTree_visitM_go___rarg___closed__4; +x_11 = l_panic___at_Lean_Elab_InfoTree_visitM_x27___spec__2___rarg(x_1, x_10); +return x_11; +} +default: +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +x_12 = lean_ctor_get(x_1, 0); +lean_inc(x_12); +lean_dec(x_1); +x_13 = lean_ctor_get(x_12, 1); +lean_inc(x_13); +lean_dec(x_12); +x_14 = lean_box(0); +x_15 = lean_apply_2(x_13, lean_box(0), x_14); +return x_15; +} +} +} +else +{ +switch (lean_obj_tag(x_5)) { +case 0: +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_5, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_5, 1); +lean_inc(x_17); +lean_dec(x_5); +x_18 = l_Lean_Elab_PartialContextInfo_mergeIntoOuter_x3f(x_16, x_4); +x_4 = x_18; +x_5 = x_17; +goto _start; +} +case 1: +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_20 = lean_ctor_get(x_4, 0); +lean_inc(x_20); +lean_dec(x_4); +x_21 = lean_ctor_get(x_5, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_5, 1); +lean_inc(x_22); +lean_dec(x_5); +x_23 = lean_ctor_get(x_1, 1); +lean_inc(x_23); +lean_inc(x_2); +lean_inc(x_22); +lean_inc(x_21); +lean_inc(x_20); +x_24 = lean_apply_3(x_2, x_20, x_21, x_22); +lean_inc(x_23); +x_25 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_visitM_x27___spec__1___rarg___lambda__1___boxed), 8, 7); +lean_closure_set(x_25, 0, x_3); +lean_closure_set(x_25, 1, x_20); +lean_closure_set(x_25, 2, x_21); +lean_closure_set(x_25, 3, x_22); +lean_closure_set(x_25, 4, x_1); +lean_closure_set(x_25, 5, x_23); +lean_closure_set(x_25, 6, x_2); +x_26 = lean_apply_4(x_23, lean_box(0), lean_box(0), x_24, x_25); +return x_26; +} +default: +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_27 = lean_ctor_get(x_1, 0); +lean_inc(x_27); +lean_dec(x_1); +x_28 = lean_ctor_get(x_27, 1); +lean_inc(x_28); +lean_dec(x_27); +x_29 = lean_box(0); +x_30 = lean_apply_2(x_28, lean_box(0), x_29); +return x_30; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_visitM_x27___spec__1(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_visitM_x27___spec__1___rarg), 5, 0); return x_2; } } @@ -985,34 +1224,44 @@ x_6 = lean_apply_3(x_1, x_2, x_3, x_4); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_5 = lean_ctor_get(x_1, 0); -lean_inc(x_5); -x_6 = lean_ctor_get(x_5, 0); +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_6 = lean_ctor_get(x_1, 0); lean_inc(x_6); -lean_dec(x_5); -x_7 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_x27___rarg___lambda__1___boxed), 5, 1); -lean_closure_set(x_7, 0, x_3); -x_8 = l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_visitM_x27___spec__1___rarg(x_1, x_2, x_7, x_4); -x_9 = lean_ctor_get(x_6, 1); -lean_inc(x_9); +x_7 = lean_ctor_get(x_6, 0); +lean_inc(x_7); lean_dec(x_6); -x_10 = lean_box(0); -x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_10, x_8); -return x_11; +x_8 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_x27___rarg___lambda__1___boxed), 5, 1); +lean_closure_set(x_8, 0, x_3); +x_9 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_visitM_x27___spec__1___rarg(x_1, x_2, x_8, x_4, x_5); +x_10 = lean_ctor_get(x_7, 1); +lean_inc(x_10); +lean_dec(x_7); +x_11 = lean_box(0); +x_12 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_11, x_9); +return x_12; } } LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_x27___rarg), 4, 0); +x_2 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_x27___rarg), 5, 0); return x_2; } } +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_visitM_x27___spec__1___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +uint8_t x_9; lean_object* x_10; +x_9 = lean_unbox(x_8); +lean_dec(x_8); +x_10 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_visitM_x27___spec__1___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_9); +return x_10; +} +} LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { @@ -1070,7 +1319,7 @@ x_2 = lean_alloc_closure((void*)(l_List_filterMapTR_go___at_Lean_Elab_InfoTree_c return x_2; } } -LEAN_EXPORT lean_object* l_List_bindTR_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__2___rarg(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__2___rarg(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -1094,15 +1343,15 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_List_bindTR_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__2(lean_object* x_1) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__2(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_List_bindTR_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__2___rarg), 2, 0); +x_2 = lean_alloc_closure((void*)(l_List_flatMapTR_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__2___rarg), 2, 0); return x_2; } } -static lean_object* _init_l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5___rarg___closed__1() { +static lean_object* _init_l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg___closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -1112,24 +1361,24 @@ x_3 = l_instInhabitedOfMonad___rarg(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5___rarg(lean_object* x_1) { +LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5___rarg___closed__1; +x_2 = l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg___closed__1; x_3 = lean_panic_fn(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5(lean_object* x_1) { +LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5___rarg), 1, 0); +x_2 = lean_alloc_closure((void*)(l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg), 1, 0); return x_2; } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__6___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { if (lean_obj_tag(x_4) == 0) @@ -1137,6 +1386,7 @@ if (lean_obj_tag(x_4) == 0) lean_object* x_6; lean_dec(x_3); lean_dec(x_2); +lean_dec(x_1); x_6 = l_List_reverse___rarg(x_5); return x_6; } @@ -1151,7 +1401,8 @@ x_8 = lean_ctor_get(x_4, 0); x_9 = lean_ctor_get(x_4, 1); lean_inc(x_3); lean_inc(x_2); -x_10 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg(x_1, x_2, x_3, x_8); +lean_inc(x_1); +x_10 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__3___rarg(x_1, x_2, x_3, x_8); lean_ctor_set(x_4, 1, x_5); lean_ctor_set(x_4, 0, x_10); { @@ -1172,7 +1423,8 @@ lean_inc(x_12); lean_dec(x_4); lean_inc(x_3); lean_inc(x_2); -x_14 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg(x_1, x_2, x_3, x_12); +lean_inc(x_1); +x_14 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__3___rarg(x_1, x_2, x_3, x_12); x_15 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_15, 0, x_14); lean_ctor_set(x_15, 1, x_5); @@ -1183,15 +1435,15 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__6(lean_object* x_1) { +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_List_mapM_loop___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__6___rarg___boxed), 5, 0); +x_2 = lean_alloc_closure((void*)(l_List_mapM_loop___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5___rarg), 5, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { if (lean_obj_tag(x_3) == 0) @@ -1215,8 +1467,9 @@ case 1: lean_object* x_9; lean_object* x_10; lean_dec(x_4); lean_dec(x_2); +lean_dec(x_1); x_9 = l_Lean_Elab_InfoTree_visitM_go___rarg___closed__4; -x_10 = l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5___rarg(x_9); +x_10 = l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg(x_9); return x_10; } default: @@ -1224,6 +1477,7 @@ return x_10; lean_object* x_11; lean_dec(x_4); lean_dec(x_2); +lean_dec(x_1); x_11 = lean_box(0); return x_11; } @@ -1251,92 +1505,117 @@ uint8_t x_16; x_16 = !lean_is_exclusive(x_3); if (x_16 == 0) { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; x_17 = lean_ctor_get(x_3, 0); x_18 = lean_ctor_get(x_4, 0); lean_inc(x_18); x_19 = lean_ctor_get(x_4, 1); lean_inc(x_19); lean_dec(x_4); +lean_inc(x_1); +lean_inc(x_19); +lean_inc(x_18); lean_inc(x_17); -x_20 = l_Lean_Elab_Info_updateContext_x3f(x_3, x_18); -x_21 = l_Lean_PersistentArray_toList___rarg(x_19); +x_20 = lean_apply_3(x_1, x_17, x_18, x_19); +x_21 = lean_unbox(x_20); +lean_dec(x_20); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; +lean_dec(x_1); x_22 = lean_box(0); +x_23 = lean_apply_4(x_2, x_17, x_18, x_19, x_22); +lean_ctor_set(x_3, 0, x_23); +return x_3; +} +else +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +lean_inc(x_17); +x_24 = l_Lean_Elab_Info_updateContext_x3f(x_3, x_18); +x_25 = l_Lean_PersistentArray_toList___rarg(x_19); +x_26 = lean_box(0); lean_inc(x_2); -x_23 = l_List_mapM_loop___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__6___rarg(x_1, x_2, x_20, x_21, x_22); -x_24 = lean_apply_4(x_2, x_17, x_18, x_19, x_23); -x_25 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_25, 0, x_24); -return x_25; +x_27 = l_List_mapM_loop___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5___rarg(x_1, x_2, x_24, x_25, x_26); +x_28 = lean_apply_4(x_2, x_17, x_18, x_19, x_27); +x_29 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_29, 0, x_28); +return x_29; +} } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_26 = lean_ctor_get(x_3, 0); -lean_inc(x_26); +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; +x_30 = lean_ctor_get(x_3, 0); +lean_inc(x_30); lean_dec(x_3); -x_27 = lean_ctor_get(x_4, 0); -lean_inc(x_27); -x_28 = lean_ctor_get(x_4, 1); -lean_inc(x_28); +x_31 = lean_ctor_get(x_4, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_4, 1); +lean_inc(x_32); lean_dec(x_4); -lean_inc(x_26); -x_29 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_29, 0, x_26); -x_30 = l_Lean_Elab_Info_updateContext_x3f(x_29, x_27); -x_31 = l_Lean_PersistentArray_toList___rarg(x_28); -x_32 = lean_box(0); +lean_inc(x_1); +lean_inc(x_32); +lean_inc(x_31); +lean_inc(x_30); +x_33 = lean_apply_3(x_1, x_30, x_31, x_32); +x_34 = lean_unbox(x_33); +lean_dec(x_33); +if (x_34 == 0) +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; +lean_dec(x_1); +x_35 = lean_box(0); +x_36 = lean_apply_4(x_2, x_30, x_31, x_32, x_35); +x_37 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_37, 0, x_36); +return x_37; +} +else +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; +lean_inc(x_30); +x_38 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_38, 0, x_30); +x_39 = l_Lean_Elab_Info_updateContext_x3f(x_38, x_31); +x_40 = l_Lean_PersistentArray_toList___rarg(x_32); +x_41 = lean_box(0); lean_inc(x_2); -x_33 = l_List_mapM_loop___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__6___rarg(x_1, x_2, x_30, x_31, x_32); -x_34 = lean_apply_4(x_2, x_26, x_27, x_28, x_33); -x_35 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_35, 0, x_34); -return x_35; +x_42 = l_List_mapM_loop___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5___rarg(x_1, x_2, x_39, x_40, x_41); +x_43 = lean_apply_4(x_2, x_30, x_31, x_32, x_42); +x_44 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_44, 0, x_43); +return x_44; +} } } default: { -lean_object* x_36; +lean_object* x_45; lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_36 = lean_box(0); -return x_36; +lean_dec(x_1); +x_45 = lean_box(0); +return x_45; } } } } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__3(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg___boxed), 4, 0); +x_2 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__3___rarg), 4, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_4; lean_object* x_5; -x_4 = lean_box(0); -x_5 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg(x_1, x_2, x_4, x_3); -return x_5; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__3(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__3___rarg___boxed), 3, 0); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = lean_box(0); +uint8_t x_4; +x_4 = 1; return x_4; } } @@ -1355,7 +1634,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___lamb lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; x_6 = l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___lambda__2___closed__1; x_7 = l_List_filterMapTR_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__1___rarg(x_5, x_6); -x_8 = l_List_bindTR_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__2___rarg(x_7, x_6); +x_8 = l_List_flatMapTR_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__2___rarg(x_7, x_6); x_9 = lean_apply_4(x_1, x_2, x_3, x_4, x_8); return x_9; } @@ -1371,24 +1650,25 @@ return x_1; LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_3; lean_object* x_4; lean_object* x_5; +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_3 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___lambda__2), 5, 1); lean_closure_set(x_3, 0, x_1); -x_4 = l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___closed__1; -x_5 = l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__3___rarg(x_4, x_3, x_2); -if (lean_obj_tag(x_5) == 0) +x_4 = lean_box(0); +x_5 = l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___closed__1; +x_6 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__3___rarg(x_5, x_3, x_4, x_2); +if (lean_obj_tag(x_6) == 0) { -lean_object* x_6; -x_6 = lean_box(0); -return x_6; +lean_object* x_7; +x_7 = lean_box(0); +return x_7; } else { -lean_object* x_7; -x_7 = lean_ctor_get(x_5, 0); -lean_inc(x_7); -lean_dec(x_5); -return x_7; +lean_object* x_8; +x_8 = lean_ctor_get(x_6, 0); +lean_inc(x_8); +lean_dec(x_6); +return x_8; } } } @@ -1400,42 +1680,16 @@ x_2 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_collectNodesBottomUp___rar return x_2; } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__6___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; -x_6 = l_List_mapM_loop___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__6___rarg(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_1); -return x_6; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -lean_object* x_5; -x_5 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg(x_1, x_2, x_3, x_4); -lean_dec(x_1); -return x_5; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__3___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__3___rarg(x_1, x_2, x_3); -lean_dec(x_1); -return x_4; -} -} LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_4; +uint8_t x_4; lean_object* x_5; x_4 = l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___lambda__1(x_1, x_2, x_3); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -return x_4; +x_5 = lean_box(x_4); +return x_5; } } LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_deepestNodes___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { @@ -6510,7 +6764,7 @@ lean_dec(x_4); return x_5; } } -LEAN_EXPORT lean_object* l_List_bindTR_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__1(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -6730,16 +6984,16 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__7(lean_object* x_1) { +LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__6(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5___rarg___closed__1; +x_2 = l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg___closed__1; x_3 = lean_panic_fn(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { if (lean_obj_tag(x_4) == 0) @@ -6747,6 +7001,7 @@ if (lean_obj_tag(x_4) == 0) lean_object* x_6; lean_dec(x_3); lean_dec(x_2); +lean_dec(x_1); x_6 = l_List_reverse___rarg(x_5); return x_6; } @@ -6761,7 +7016,8 @@ x_8 = lean_ctor_get(x_4, 0); x_9 = lean_ctor_get(x_4, 1); lean_inc(x_3); lean_inc(x_2); -x_10 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__6(x_1, x_2, x_3, x_8); +lean_inc(x_1); +x_10 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__5(x_1, x_2, x_3, x_8); lean_ctor_set(x_4, 1, x_5); lean_ctor_set(x_4, 0, x_10); { @@ -6782,7 +7038,8 @@ lean_inc(x_12); lean_dec(x_4); lean_inc(x_3); lean_inc(x_2); -x_14 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__6(x_1, x_2, x_3, x_12); +lean_inc(x_1); +x_14 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__5(x_1, x_2, x_3, x_12); x_15 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_15, 0, x_14); lean_ctor_set(x_15, 1, x_5); @@ -6793,7 +7050,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { if (lean_obj_tag(x_3) == 0) @@ -6817,8 +7074,9 @@ case 1: lean_object* x_9; lean_object* x_10; lean_dec(x_4); lean_dec(x_2); +lean_dec(x_1); x_9 = l_Lean_Elab_InfoTree_visitM_go___rarg___closed__4; -x_10 = l_panic___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__7(x_9); +x_10 = l_panic___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__6(x_9); return x_10; } default: @@ -6826,6 +7084,7 @@ return x_10; lean_object* x_11; lean_dec(x_4); lean_dec(x_2); +lean_dec(x_1); x_11 = lean_box(0); return x_11; } @@ -6853,72 +7112,105 @@ uint8_t x_16; x_16 = !lean_is_exclusive(x_3); if (x_16 == 0) { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; x_17 = lean_ctor_get(x_3, 0); x_18 = lean_ctor_get(x_4, 0); lean_inc(x_18); x_19 = lean_ctor_get(x_4, 1); lean_inc(x_19); lean_dec(x_4); +lean_inc(x_1); +lean_inc(x_19); +lean_inc(x_18); lean_inc(x_17); -x_20 = l_Lean_Elab_Info_updateContext_x3f(x_3, x_18); -x_21 = l_Lean_PersistentArray_toList___rarg(x_19); +x_20 = lean_apply_3(x_1, x_17, x_18, x_19); +x_21 = lean_unbox(x_20); +lean_dec(x_20); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; +lean_dec(x_1); x_22 = lean_box(0); +x_23 = lean_apply_4(x_2, x_17, x_18, x_19, x_22); +lean_ctor_set(x_3, 0, x_23); +return x_3; +} +else +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +lean_inc(x_17); +x_24 = l_Lean_Elab_Info_updateContext_x3f(x_3, x_18); +x_25 = l_Lean_PersistentArray_toList___rarg(x_19); +x_26 = lean_box(0); lean_inc(x_2); -x_23 = l_List_mapM_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8(x_1, x_2, x_20, x_21, x_22); -x_24 = lean_apply_4(x_2, x_17, x_18, x_19, x_23); -x_25 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_25, 0, x_24); -return x_25; +x_27 = l_List_mapM_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__7(x_1, x_2, x_24, x_25, x_26); +x_28 = lean_apply_4(x_2, x_17, x_18, x_19, x_27); +x_29 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_29, 0, x_28); +return x_29; +} } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_26 = lean_ctor_get(x_3, 0); -lean_inc(x_26); +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; +x_30 = lean_ctor_get(x_3, 0); +lean_inc(x_30); lean_dec(x_3); -x_27 = lean_ctor_get(x_4, 0); -lean_inc(x_27); -x_28 = lean_ctor_get(x_4, 1); -lean_inc(x_28); +x_31 = lean_ctor_get(x_4, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_4, 1); +lean_inc(x_32); lean_dec(x_4); -lean_inc(x_26); -x_29 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_29, 0, x_26); -x_30 = l_Lean_Elab_Info_updateContext_x3f(x_29, x_27); -x_31 = l_Lean_PersistentArray_toList___rarg(x_28); -x_32 = lean_box(0); +lean_inc(x_1); +lean_inc(x_32); +lean_inc(x_31); +lean_inc(x_30); +x_33 = lean_apply_3(x_1, x_30, x_31, x_32); +x_34 = lean_unbox(x_33); +lean_dec(x_33); +if (x_34 == 0) +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; +lean_dec(x_1); +x_35 = lean_box(0); +x_36 = lean_apply_4(x_2, x_30, x_31, x_32, x_35); +x_37 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_37, 0, x_36); +return x_37; +} +else +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; +lean_inc(x_30); +x_38 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_38, 0, x_30); +x_39 = l_Lean_Elab_Info_updateContext_x3f(x_38, x_31); +x_40 = l_Lean_PersistentArray_toList___rarg(x_32); +x_41 = lean_box(0); lean_inc(x_2); -x_33 = l_List_mapM_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8(x_1, x_2, x_30, x_31, x_32); -x_34 = lean_apply_4(x_2, x_26, x_27, x_28, x_33); -x_35 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_35, 0, x_34); -return x_35; +x_42 = l_List_mapM_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__7(x_1, x_2, x_39, x_40, x_41); +x_43 = lean_apply_4(x_2, x_30, x_31, x_32, x_42); +x_44 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_44, 0, x_43); +return x_44; +} } } default: { -lean_object* x_36; +lean_object* x_45; lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_36 = lean_box(0); -return x_36; -} -} +lean_dec(x_1); +x_45 = lean_box(0); +return x_45; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; lean_object* x_5; -x_4 = lean_box(0); -x_5 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__6(x_1, x_2, x_4, x_3); -return x_5; } } -LEAN_EXPORT uint8_t l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_5; uint8_t x_6; @@ -6955,7 +7247,7 @@ return x_10; } } } -LEAN_EXPORT uint8_t l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__11(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_5; uint8_t x_6; @@ -6992,7 +7284,7 @@ return x_10; } } } -LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___lambda__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___lambda__1(lean_object* x_1) { _start: { lean_object* x_2; @@ -7001,7 +7293,7 @@ lean_inc(x_2); return x_2; } } -LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___lambda__2(lean_object* x_1) { +LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___lambda__2(lean_object* x_1) { _start: { lean_object* x_2; @@ -7010,31 +7302,31 @@ lean_inc(x_2); return x_2; } } -static lean_object* _init_l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___closed__1() { +static lean_object* _init_l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___lambda__1___boxed), 1, 0); +x_1 = lean_alloc_closure((void*)(l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___lambda__1___boxed), 1, 0); return x_1; } } -static lean_object* _init_l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___closed__2() { +static lean_object* _init_l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___closed__2() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___lambda__2___boxed), 1, 0); +x_1 = lean_alloc_closure((void*)(l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___lambda__2___boxed), 1, 0); return x_1; } } -static lean_object* _init_l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9() { +static lean_object* _init_l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___closed__1; -x_2 = lean_alloc_closure((void*)(l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__10___boxed), 3, 1); +x_1 = l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___closed__1; +x_2 = lean_alloc_closure((void*)(l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___boxed), 3, 1); lean_closure_set(x_2, 0, x_1); -x_3 = l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___closed__2; -x_4 = lean_alloc_closure((void*)(l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__11___boxed), 3, 1); +x_3 = l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___closed__2; +x_4 = lean_alloc_closure((void*)(l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__10___boxed), 3, 1); lean_closure_set(x_4, 0, x_3); x_5 = lean_alloc_closure((void*)(l_lexOrd___elambda__1___rarg), 4, 2); lean_closure_set(x_5, 0, x_2); @@ -7042,7 +7334,7 @@ lean_closure_set(x_5, 1, x_4); return x_5; } } -LEAN_EXPORT uint8_t l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__13(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__12(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_5; uint8_t x_6; @@ -7079,27 +7371,27 @@ return x_10; } } } -LEAN_EXPORT lean_object* l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__14(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__13(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_inc(x_1); x_4 = lean_apply_1(x_1, x_2); x_5 = lean_apply_1(x_1, x_3); -x_6 = l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9; +x_6 = l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8; x_7 = lean_apply_2(x_6, x_4, x_5); return x_7; } } -static lean_object* _init_l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__12() { +static lean_object* _init_l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___closed__1; -x_2 = lean_alloc_closure((void*)(l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__13___boxed), 3, 1); +x_1 = l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___closed__1; +x_2 = lean_alloc_closure((void*)(l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__12___boxed), 3, 1); lean_closure_set(x_2, 0, x_1); -x_3 = l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___closed__2; -x_4 = lean_alloc_closure((void*)(l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__14), 3, 1); +x_3 = l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___closed__2; +x_4 = lean_alloc_closure((void*)(l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__13), 3, 1); lean_closure_set(x_4, 0, x_3); x_5 = lean_alloc_closure((void*)(l_lexOrd___elambda__1___rarg), 4, 2); lean_closure_set(x_5, 0, x_2); @@ -7107,7 +7399,7 @@ lean_closure_set(x_5, 1, x_4); return x_5; } } -LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__15(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__14(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -7159,7 +7451,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__17(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__16(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { if (lean_obj_tag(x_4) == 0) @@ -7195,7 +7487,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__16(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__15(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_3) == 0) @@ -7213,14 +7505,14 @@ lean_inc(x_5); x_6 = lean_ctor_get(x_3, 1); lean_inc(x_6); lean_dec(x_3); -x_7 = l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__17(x_1, x_2, x_5, x_6); +x_7 = l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__16(x_1, x_2, x_5, x_6); x_8 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_8, 0, x_7); return x_8; } } } -LEAN_EXPORT uint8_t l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__18(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__17(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -7287,7 +7579,7 @@ return x_20; } } } -LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__20(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__19(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { if (lean_obj_tag(x_4) == 0) @@ -7323,7 +7615,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__19(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__18(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_3) == 0) @@ -7341,7 +7633,7 @@ lean_inc(x_5); x_6 = lean_ctor_get(x_3, 1); lean_inc(x_6); lean_dec(x_3); -x_7 = l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__20(x_1, x_2, x_5, x_6); +x_7 = l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__19(x_1, x_2, x_5, x_6); x_8 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_8, 0, x_7); return x_8; @@ -7827,7 +8119,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__7(le lean_object* x_9; lean_object* x_10; lean_object* x_11; x_9 = lean_box(0); x_10 = l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___lambda__2___closed__1; -x_11 = l_List_bindTR_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__1(x_8, x_10); +x_11 = l_List_flatMapTR_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__1(x_8, x_10); if (x_4 == 0) { lean_object* x_12; lean_object* x_13; @@ -7885,7 +8177,7 @@ x_3 = lean_ctor_get(x_2, 0); lean_inc(x_3); x_4 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_4, 0, x_3); -x_5 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__18(x_4, x_1); +x_5 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__17(x_4, x_1); lean_dec(x_4); return x_5; } @@ -7893,7 +8185,7 @@ return x_5; LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, uint8_t x_5) { _start: { -lean_object* x_6; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +lean_object* x_6; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; x_14 = lean_box(x_3); x_15 = lean_box(x_5); x_16 = lean_box(x_4); @@ -7902,47 +8194,46 @@ lean_closure_set(x_17, 0, x_2); lean_closure_set(x_17, 1, x_14); lean_closure_set(x_17, 2, x_15); lean_closure_set(x_17, 3, x_16); -x_18 = l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___closed__1; -x_19 = l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__5(x_18, x_17, x_1); -x_20 = lean_box(0); +x_18 = lean_box(0); +x_19 = l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___closed__1; +x_20 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__5(x_19, x_17, x_18, x_1); x_21 = lean_box(0); -if (lean_obj_tag(x_19) == 0) +x_22 = lean_box(0); +if (lean_obj_tag(x_20) == 0) { -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_22 = l_List_mapTR_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__15(x_21, x_21); -x_23 = l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__12; -x_24 = l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__16(x_23, x_20, x_22); -x_25 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__8___boxed), 2, 1); -lean_closure_set(x_25, 0, x_24); -x_26 = l_List_find_x3f___rarg(x_25, x_21); -if (lean_obj_tag(x_26) == 0) +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_23 = l_List_mapTR_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__14(x_22, x_22); +x_24 = l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__11; +x_25 = l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__15(x_24, x_21, x_23); +x_26 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__8___boxed), 2, 1); +lean_closure_set(x_26, 0, x_25); +x_27 = l_List_find_x3f___rarg(x_26, x_22); +if (lean_obj_tag(x_27) == 0) { -lean_object* x_27; -x_27 = lean_box(0); -x_6 = x_27; +x_6 = x_18; goto block_13; } else { uint8_t x_28; -x_28 = !lean_is_exclusive(x_26); +x_28 = !lean_is_exclusive(x_27); if (x_28 == 0) { lean_object* x_29; lean_object* x_30; -x_29 = lean_ctor_get(x_26, 0); +x_29 = lean_ctor_get(x_27, 0); x_30 = lean_ctor_get(x_29, 1); lean_inc(x_30); lean_dec(x_29); -lean_ctor_set(x_26, 0, x_30); -x_6 = x_26; +lean_ctor_set(x_27, 0, x_30); +x_6 = x_27; goto block_13; } else { lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_31 = lean_ctor_get(x_26, 0); +x_31 = lean_ctor_get(x_27, 0); lean_inc(x_31); -lean_dec(x_26); +lean_dec(x_27); x_32 = lean_ctor_get(x_31, 1); lean_inc(x_32); lean_dec(x_31); @@ -7956,50 +8247,48 @@ goto block_13; else { lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_34 = lean_ctor_get(x_19, 0); +x_34 = lean_ctor_get(x_20, 0); lean_inc(x_34); -lean_dec(x_19); +lean_dec(x_20); lean_inc(x_34); -x_35 = l_List_mapTR_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__15(x_34, x_21); -x_36 = l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__12; -x_37 = l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__19(x_36, x_20, x_35); +x_35 = l_List_mapTR_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__14(x_34, x_22); +x_36 = l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__11; +x_37 = l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__18(x_36, x_21, x_35); x_38 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__8___boxed), 2, 1); lean_closure_set(x_38, 0, x_37); x_39 = l_List_find_x3f___rarg(x_38, x_34); if (lean_obj_tag(x_39) == 0) { -lean_object* x_40; -x_40 = lean_box(0); -x_6 = x_40; +x_6 = x_18; goto block_13; } else { -uint8_t x_41; -x_41 = !lean_is_exclusive(x_39); -if (x_41 == 0) +uint8_t x_40; +x_40 = !lean_is_exclusive(x_39); +if (x_40 == 0) { -lean_object* x_42; lean_object* x_43; -x_42 = lean_ctor_get(x_39, 0); -x_43 = lean_ctor_get(x_42, 1); -lean_inc(x_43); -lean_dec(x_42); -lean_ctor_set(x_39, 0, x_43); +lean_object* x_41; lean_object* x_42; +x_41 = lean_ctor_get(x_39, 0); +x_42 = lean_ctor_get(x_41, 1); +lean_inc(x_42); +lean_dec(x_41); +lean_ctor_set(x_39, 0, x_42); x_6 = x_39; goto block_13; } else { -lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_44 = lean_ctor_get(x_39, 0); -lean_inc(x_44); +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_39, 0); +lean_inc(x_43); lean_dec(x_39); -x_45 = lean_ctor_get(x_44, 1); -lean_inc(x_45); -lean_dec(x_44); -x_46 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_46, 0, x_45); -x_6 = x_46; +x_44 = lean_ctor_get(x_43, 1); +lean_inc(x_44); +lean_dec(x_43); +x_45 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_45, 0, x_44); +x_6 = x_45; goto block_13; } } @@ -8050,121 +8339,94 @@ return x_6; } } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; -x_6 = l_List_mapM_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_1); -return x_6; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -lean_object* x_5; -x_5 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__6(x_1, x_2, x_3, x_4); -lean_dec(x_1); -return x_5; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__5(x_1, x_2, x_3); -lean_dec(x_1); -return x_4; -} -} -LEAN_EXPORT lean_object* l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; -x_4 = l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__10(x_1, x_2, x_3); +x_4 = l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9(x_1, x_2, x_3); x_5 = lean_box(x_4); return x_5; } } -LEAN_EXPORT lean_object* l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; -x_4 = l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__11(x_1, x_2, x_3); +x_4 = l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__10(x_1, x_2, x_3); x_5 = lean_box(x_4); return x_5; } } -LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___lambda__1___boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___lambda__1___boxed(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___lambda__1(x_1); +x_2 = l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___lambda__1(x_1); lean_dec(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___lambda__2___boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___lambda__2___boxed(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___lambda__2(x_1); +x_2 = l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___lambda__2(x_1); lean_dec(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__12___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; -x_4 = l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__13(x_1, x_2, x_3); +x_4 = l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__12(x_1, x_2, x_3); x_5 = lean_box(x_4); return x_5; } } -LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__17___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__16___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__17(x_1, x_2, x_3, x_4); +x_5 = l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__16(x_1, x_2, x_3, x_4); lean_dec(x_2); return x_5; } } -LEAN_EXPORT lean_object* l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__16___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__15___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__16(x_1, x_2, x_3); +x_4 = l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__15(x_1, x_2, x_3); lean_dec(x_2); return x_4; } } -LEAN_EXPORT lean_object* l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__18___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__17___boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__18(x_1, x_2); +x_3 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__17(x_1, x_2); lean_dec(x_2); lean_dec(x_1); x_4 = lean_box(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__20___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__19___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__20(x_1, x_2, x_3, x_4); +x_5 = l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__19(x_1, x_2, x_3, x_4); lean_dec(x_2); return x_5; } } -LEAN_EXPORT lean_object* l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__19___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__18___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__19(x_1, x_2, x_3); +x_4 = l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__18(x_1, x_2, x_3); lean_dec(x_2); return x_4; } @@ -19514,8 +19776,8 @@ l_Lean_Elab_InfoTree_visitM_go___rarg___closed__3 = _init_l_Lean_Elab_InfoTree_v lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___rarg___closed__3); l_Lean_Elab_InfoTree_visitM_go___rarg___closed__4 = _init_l_Lean_Elab_InfoTree_visitM_go___rarg___closed__4(); lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___rarg___closed__4); -l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5___rarg___closed__1 = _init_l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5___rarg___closed__1(); -lean_mark_persistent(l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5___rarg___closed__1); +l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg___closed__1 = _init_l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg___closed__1(); +lean_mark_persistent(l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg___closed__1); l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___lambda__2___closed__1 = _init_l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___lambda__2___closed__1(); lean_mark_persistent(l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___lambda__2___closed__1); l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___closed__1 = _init_l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___closed__1(); @@ -19532,14 +19794,14 @@ l_List_mapTR_loop___at_Lean_Elab_InfoTree_smallestInfo_x3f___spec__1___closed__3 lean_mark_persistent(l_List_mapTR_loop___at_Lean_Elab_InfoTree_smallestInfo_x3f___spec__1___closed__3); l_List_mapTR_loop___at_Lean_Elab_InfoTree_smallestInfo_x3f___spec__1___closed__4 = _init_l_List_mapTR_loop___at_Lean_Elab_InfoTree_smallestInfo_x3f___spec__1___closed__4(); lean_mark_persistent(l_List_mapTR_loop___at_Lean_Elab_InfoTree_smallestInfo_x3f___spec__1___closed__4); -l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___closed__1 = _init_l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___closed__1(); -lean_mark_persistent(l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___closed__1); -l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___closed__2 = _init_l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___closed__2(); -lean_mark_persistent(l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___closed__2); -l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9 = _init_l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9(); -lean_mark_persistent(l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9); -l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__12 = _init_l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__12(); -lean_mark_persistent(l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__12); +l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___closed__1 = _init_l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___closed__1(); +lean_mark_persistent(l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___closed__1); +l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___closed__2 = _init_l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___closed__2(); +lean_mark_persistent(l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___closed__2); +l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8 = _init_l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8(); +lean_mark_persistent(l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8); +l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__11 = _init_l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__11(); +lean_mark_persistent(l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__11); l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__4___closed__1 = _init_l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__4___closed__1(); lean_mark_persistent(l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__4___closed__1); l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__4___closed__2 = _init_l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__4___closed__2(); diff --git a/stage0/stdlib/Lean/Server/References.c b/stage0/stdlib/Lean/Server/References.c index e74881e3b117..eace061f0f84 100644 --- a/stage0/stdlib/Lean/Server/References.c +++ b/stage0/stdlib/Lean/Server/References.c @@ -20,13 +20,11 @@ lean_object* l_Lean_JsonNumber_fromNat(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_findReferences___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_findDeclarationRanges_x3f___at_Lean_Server_RefInfo_toLspRefInfo___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Lsp_RefIdent_toJson(lean_object*); -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Server_combineIdents_buildIdMap___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_References_definitionsMatching___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterTR_loop___at_Lean_Server_References_removeIlean___spec__3(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonRpcCallParams____x40_Lean_Data_Lsp_Extra___hyg_2012____spec__1(lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_References_allRefsFor___spec__3___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_combineIdents_useConstRepresentatives___spec__26(size_t, lean_object*, lean_object*, size_t, size_t, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___closed__1; LEAN_EXPORT lean_object* l_Lean_Lsp_RefInfo_empty; lean_object* l_instBEqOfDecidableEq___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_References_allRefs___spec__6___boxed(lean_object*, lean_object*); @@ -35,6 +33,7 @@ lean_object* l_Lean_Json_compress(lean_object*); static lean_object* l___private_Lean_Server_References_0__Lean_Server_fromJsonIlean____x40_Lean_Server_References___hyg_1333____closed__1; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_References_addIlean___spec__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_isRec___at_Lean_Server_RefInfo_toLspRefInfo___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_IO_throwServerError___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_References_findAt(lean_object*, lean_object*, lean_object*, uint8_t); uint8_t l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_beqRange____x40_Lean_Data_Lsp_Basic___hyg_627_(lean_object*, lean_object*); @@ -43,6 +42,7 @@ uint64_t l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_hashRefIdent____x40_Lean LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_References_allRefs___spec__10(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_References_allRefsFor___spec__5(lean_object*, size_t, size_t, lean_object*); static lean_object* l_List_mapTR_loop___at___private_Lean_Server_References_0__Lean_Server_toJsonIlean____x40_Lean_Server_References___hyg_1478____spec__2___closed__3; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Server_References_allRefs___spec__3(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_dedupReferences___closed__2; static lean_object* l_Lean_Server_findModuleRefs___closed__2; @@ -50,14 +50,15 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Ser LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_combineIdents_useConstRepresentatives___spec__24(size_t, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Server_References_removeWorkerRefs___spec__1___boxed(lean_object*, lean_object*); lean_object* l_Lean_Json_mkObj(lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__7___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_declRangeExt; static lean_object* l_Lean_Server_dedupReferences___closed__11; -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_combineIdents_useConstRepresentatives___spec__23(size_t, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_dedupReferences(lean_object*, uint8_t); static lean_object* l_Lean_Server_dedupReferences___closed__10; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_References_definitionsMatching___spec__5(lean_object*, size_t, size_t, lean_object*); lean_object* l_Lean_Syntax_getHeadInfo(lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Server_ModuleRefs_addRef___spec__6(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_References_allRefs___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Server_References_updateWorkerRefs___spec__6(lean_object*, lean_object*, lean_object*); @@ -91,7 +92,6 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Ser lean_object* l_Array_qpartition___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_References_definitionOf_x3f___spec__1(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Server_References_allRefsFor___spec__7___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Server_combineIdents_buildIdMap___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_RefInfo_toLspRefInfo___spec__6___closed__3; lean_object* lean_mk_array(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Server_combineIdents_buildIdMap___spec__1___boxed(lean_object*, lean_object*); @@ -107,20 +107,19 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_findModuleRe static lean_object* l_Array_qsort_sort___at_Lean_Server_dedupReferences___spec__10___closed__1; static lean_object* l_Lean_Server_dedupReferences___closed__6; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_RefInfo_toLspRefInfo___spec__6(size_t, size_t, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_panic___at_Lean_Server_combineIdents_buildIdMap___spec__6(lean_object*, lean_object*); extern lean_object* l_Lean_Lsp_instOrdPosition; lean_object* lean_array_fget(lean_object*, lean_object*); lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_References_definitionsMatching___spec__2(lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_combineIdents___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_References_removeIlean___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_References_0__Lean_Server_fromJsonIlean____x40_Lean_Server_References___hyg_1333____closed__5; -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Server_dedupReferences___spec__10(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Server_combineIdents_useConstRepresentatives___spec__12(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_combineIdents_useConstRepresentatives___spec__6(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_dedupReferences___spec__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_References_allRefs___spec__6(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_References_allRefs___spec__11(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Lsp_ModuleRefs_findRange_x3f___spec__3(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); @@ -129,19 +128,20 @@ lean_object* l_System_Uri_pathToUri(lean_object*); LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Server_ModuleRefs_toLspModuleRefs___spec__2(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_combineIdents_useConstRepresentatives___spec__9(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Lsp_ModuleRefs_findAt___spec__2(lean_object*, uint8_t, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_combineIdents_useConstRepresentatives___spec__21(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_combineIdents_useConstRepresentatives___spec__18(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_References_findRange_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Lsp_ModuleRefs_findRange_x3f___spec__1(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_References_0__Lean_Server_toJsonIlean____x40_Lean_Server_References___hyg_1478____spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_References_allRefsFor___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Nat_nextPowerOfTwo_go(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_combineIdents_buildIdMap___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_combineIdents_buildIdMap___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_instDecidableRelLt___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_ModuleRefs_findRange_x3f___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Server_References_removeIlean___spec__4(lean_object*, lean_object*); static lean_object* l_Lean_Lsp_RefInfo_findReferenceLocation_x3f___lambda__2___closed__1; +lean_object* l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_References_0__Lean_Server_fromJsonIlean____x40_Lean_Server_References___hyg_1333____closed__14; lean_object* l_EStateM_instMonad(lean_object*, lean_object*); lean_object* l_Lean_PersistentArray_toList___rarg(lean_object*); @@ -175,19 +175,19 @@ LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_References_definitio lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_References_0__Lean_Server_fromJsonIlean____x40_Lean_Server_References___hyg_1333____closed__6; LEAN_EXPORT lean_object* l_Lean_Server_findModuleRefs(lean_object*, lean_object*, uint8_t, uint8_t); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_appendTR___rarg(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__1; LEAN_EXPORT uint8_t l_Array_qsort_sort___at_Lean_Server_dedupReferences___spec__10___lambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_References_definitionsMatching___spec__6___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_instToJsonIlean___closed__1; size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_findModuleRefs___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Server_combineIdents_buildIdMap___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_TagDeclarationExtension_isTagged(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_findModuleRefs___lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_References_findAt___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Lsp_ModuleRefs_findAt___spec__4(lean_object*, size_t, size_t, lean_object*); -static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__1; LEAN_EXPORT lean_object* l_Lean_Lsp_ModuleRefs_findAt(lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_combineIdents_useConstRepresentatives___spec__22___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_RefInfo_findReferenceLocation_x3f(lean_object*, lean_object*, uint8_t); @@ -195,18 +195,19 @@ LEAN_EXPORT lean_object* l_Lean_Lsp_RefInfo_contains___boxed(lean_object*, lean_ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Server_combineIdents_useConstRepresentatives___spec__12___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_References_definitionsMatching(lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Lsp_ModuleRefs_findRange_x3f___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_findReferences___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_findReferences___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at_Lean_Server_combineIdents_findCanonicalRepresentative___spec__3(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_findDeclarationRangesCore_x3f___at_Lean_Server_RefInfo_toLspRefInfo___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_References_empty; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_combineIdents___spec__6(lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l___private_Lean_Server_References_0__Lean_Server_fromJsonIlean____x40_Lean_Server_References___hyg_1333____closed__17; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_References_allRefsFor___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_panic___at_Lean_Server_findReferences___spec__4___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_combineIdents_buildIdMap___spec__2(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Server_References_0__Lean_Server_toJsonIlean____x40_Lean_Server_References___hyg_1478____spec__2(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_References_finalizeWorkerRefs___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_combineIdents_buildIdMap___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Server_References_updateWorkerRefs___spec__9___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_panic___at_Lean_Server_findReferences___spec__3___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_References_removeIlean___spec__7(lean_object*, size_t, size_t, lean_object*); uint64_t lean_uint64_shift_right(uint64_t, uint64_t); static uint64_t l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_dedupReferences___spec__4___at_Lean_Server_dedupReferences___spec__5___closed__2; @@ -260,6 +261,7 @@ lean_object* l_instDecidableEqBool___boxed(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_References_allRefs___spec__1(lean_object*, lean_object*); static lean_object* l_List_mapTR_loop___at___private_Lean_Server_References_0__Lean_Server_toJsonIlean____x40_Lean_Server_References___hyg_1478____spec__2___closed__2; static lean_object* l_Lean_Server_dedupReferences___closed__4; +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__4; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_References_definitionsMatching___spec__3(lean_object*); static lean_object* l___private_Lean_Server_References_0__Lean_Server_fromJsonIlean____x40_Lean_Server_References___hyg_1333____closed__16; LEAN_EXPORT lean_object* l_Lean_Server_combineIdents_findCanonicalRepresentative(lean_object*, lean_object*); @@ -283,7 +285,9 @@ static lean_object* l_Lean_Server_ModuleRefs_toLspModuleRefs___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_combineIdents_useConstRepresentatives___spec__26___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_References_definitionOf_x3f___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_References_allRefsFor___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__7(lean_object*, size_t, size_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_References_updateWorkerRefs___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__2; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Lsp_ModuleRefs_findRange_x3f___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_ModuleRefs_toLspModuleRefs___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_ModuleRefs_toLspModuleRefs___spec__1(lean_object*, lean_object*); @@ -299,7 +303,6 @@ lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l_Lean_Server_Ilean_load___closed__2; lean_object* l_Lean_MapDeclarationExtension_find_x3f___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_RefInfo_addRef(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_panic___at_Lean_Server_findReferences___spec__4(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_findReferences___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Server_References_allRefs___spec__5(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_References_allRefs___spec__4(lean_object*, lean_object*); @@ -309,6 +312,7 @@ LEAN_EXPORT lean_object* l_Lean_Server_Ilean_load(lean_object*, lean_object*); extern lean_object* l_instMonadBaseIO; static size_t l_Lean_Server_References_allRefsFor___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_combineIdents___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_panic___at_Lean_Server_combineIdents_buildIdMap___spec__5(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_forInStep_go___at_Lean_Server_combineIdents_useConstRepresentatives___spec__14(lean_object*, lean_object*); lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Lsp_RefInfo_empty___closed__1; @@ -321,7 +325,6 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_References_re LEAN_EXPORT lean_object* l_List_filterTR_loop___at_Lean_Server_References_removeIlean___spec__3___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Server_combineIdents_buildIdMap___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Server_ModuleRefs_addRef___spec__1___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Server_findReferences___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_References_allRefsFor___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_forInStep_go___at_Lean_Server_combineIdents_useConstRepresentatives___spec__20(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_References_addIlean___spec__2(lean_object*); @@ -341,15 +344,14 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get___at_Lean_Server_ LEAN_EXPORT lean_object* l_Lean_Server_ModuleRefs_toLspModuleRefs(lean_object*, lean_object*); extern lean_object* l_Lean_Lsp_instHashableRefIdent; static lean_object* l___private_Lean_Server_References_0__Lean_Server_fromJsonIlean____x40_Lean_Server_References___hyg_1333____closed__21; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_getModuleContainingDecl_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_References_allRefs___spec__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Server_References_removeIlean___spec__5(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_References_allRefs(lean_object*); -lean_object* l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_RefInfo_toLspRefInfo___spec__6___closed__2; lean_object* l_IO_FS_readFile(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_References_addIlean___spec__4(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8(lean_object*, size_t, size_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_ModuleRefs_toLspModuleRefs___spec__4(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_References_0__Lean_Server_toJsonIlean____x40_Lean_Server_References___hyg_1478_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_References_definitionOf_x3f(lean_object*, lean_object*, lean_object*, lean_object*); @@ -359,11 +361,9 @@ LEAN_EXPORT lean_object* l_Lean_findDeclarationRanges_x3f___at_Lean_Server_RefIn static lean_object* l___private_Lean_Server_References_0__Lean_Server_fromJsonIlean____x40_Lean_Server_References___hyg_1333____closed__4; LEAN_EXPORT lean_object* l_Lean_Server_combineIdents_useConstRepresentatives(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_combineIdents_buildIdMap(lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8___closed__1; LEAN_EXPORT lean_object* l_Lean_Server_References_findAt___lambda__1___boxed(lean_object*); lean_object* l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_References_definitionsMatching___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_panic___at_Lean_Server_findReferences___spec__4___closed__2; lean_object* l_StateT_instMonad___rarg(lean_object*); lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_instRpcEncodableArray___spec__2(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_combineIdents_findCanonicalRepresentative___boxed(lean_object*, lean_object*); @@ -378,6 +378,7 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdent LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_ModuleRefs_toLspModuleRefs___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_combineIdents_findCanonicalRepresentative___spec__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at_Lean_Server_combineIdents_findCanonicalRepresentative___spec__3___boxed(lean_object*, lean_object*); +static lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__7___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_useConstRepresentatives___spec__27___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_combineIdents_useConstRepresentatives___spec__1___boxed(lean_object*, lean_object*); lean_object* l_Std_Internal_Parsec_String_Parser_run___rarg(lean_object*, lean_object*); @@ -388,6 +389,7 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Ser LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Server_References_allRefsFor___spec__7(lean_object*, lean_object*); static lean_object* l_Lean_Server_References_findAt___closed__1; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Server_dedupReferences___spec__7(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__7___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_References_0__Lean_Server_fromJsonIlean____x40_Lean_Server_References___hyg_1333____closed__18; uint8_t l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_Lean_PrettyPrinter_delabCore___spec__3(lean_object*, lean_object*); @@ -424,7 +426,6 @@ static lean_object* l_Lean_Server_dedupReferences___closed__1; extern lean_object* l_Lean_Lsp_instBEqRefIdent; lean_object* lean_panic_fn(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_dedupReferences___spec__4(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Lsp_ModuleRefs_findAt___spec__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_References_definitionsMatching___spec__1___boxed(lean_object*, lean_object*); @@ -432,11 +433,8 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_References_a lean_object* lean_nat_mul(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_RefInfo_findReferenceLocation_x3f___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_References_0__Lean_Server_fromJsonIlean____x40_Lean_Server_References___hyg_1333____closed__22; -static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__2; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Server_combineIdents_useConstRepresentatives___spec__2(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_ModuleRefs_toLspModuleRefs___closed__3; -static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__3; -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Server_findReferences___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_ModuleRefs_addRef___spec__3(lean_object*); lean_object* l_Lean_Elab_Info_range_x3f(lean_object*); lean_object* l_Lean_Json_Parser_any(lean_object*); @@ -452,12 +450,15 @@ lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Position_0__Le lean_object* l_List_reverse___rarg(lean_object*); lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Lsp_instFromJsonModuleRefs___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_combineIdents_useConstRepresentatives___spec__15(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Server_findReferences___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Server_combineIdents_useConstRepresentatives___spec__5(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_References_definitionsMatching___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterTR_loop___at_Lean_Server_References_removeIlean___spec__6(lean_object*, lean_object*, lean_object*); size_t lean_usize_sub(size_t, size_t); lean_object* lean_array_mk(lean_object*); +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__3; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Server_References_updateWorkerRefs___spec__2___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_panic___at_Lean_Server_findReferences___spec__3(lean_object*, lean_object*); extern lean_object* l_Lean_noConfusionExt; uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Lsp_instFromJsonModuleRefs___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_combineIdents_useConstRepresentatives___spec__21___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -465,13 +466,11 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_RefInfo_toLspRe static lean_object* l_Lean_Server_ModuleRefs_toLspModuleRefs___closed__2; static lean_object* l_Lean_Server_Ilean_load___closed__1; size_t lean_usize_add(size_t, size_t); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_ReaderT_pure___at_Lean_Server_RefInfo_toLspRefInfo___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_References_updateWorkerRefs___spec__4___boxed(lean_object*, lean_object*); static lean_object* l_List_mapTR_loop___at___private_Lean_Server_References_0__Lean_Server_toJsonIlean____x40_Lean_Server_References___hyg_1478____spec__2___closed__1; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_combineIdents___spec__4(lean_object*, lean_object*); lean_object* lean_array_uget(lean_object*, size_t); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_array_size(lean_object*); LEAN_EXPORT lean_object* l_List_filterTR_loop___at_Lean_Server_References_removeIlean___spec__6___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_References_0__Lean_Server_fromJsonIlean____x40_Lean_Server_References___hyg_1333____closed__15; @@ -498,7 +497,6 @@ LEAN_EXPORT lean_object* l_Lean_Server_References_finalizeWorkerRefs(lean_object LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Server_References_addIlean___spec__3(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_combineIdents_useConstRepresentatives___spec__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); -static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__4; LEAN_EXPORT lean_object* l_Lean_Lsp_RefInfo_findReferenceLocation_x3f___lambda__2(lean_object*, lean_object*, uint8_t, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_References_allRefsFor___spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_ModuleRefs_addRef___spec__2___boxed(lean_object*, lean_object*); @@ -519,15 +517,14 @@ LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_ LEAN_EXPORT lean_object* l_Lean_Server_References_allRefs___boxed(lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_RefInfo_toLspRefInfo___spec__6___closed__5; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_combineIdents___spec__7(lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_combineIdents_buildIdMap___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterTR_loop___at_Lean_Server_References_removeIlean___spec__8___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_References_updateWorkerRefs___spec__3(uint64_t, uint64_t, size_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_combineIdents___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_instToJsonIlean; static lean_object* l___private_Lean_Server_References_0__Lean_Server_fromJsonIlean____x40_Lean_Server_References___hyg_1333____closed__12; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_combineIdents_useConstRepresentatives___spec__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_References_allRefs___spec__7(lean_object*, lean_object*); +static lean_object* l_panic___at_Lean_Server_findReferences___spec__3___closed__2; LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_References_addIlean___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_References_definitionsMatching___spec__4___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_References_updateWorkerRefs___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, uint64_t, uint64_t, size_t, lean_object*); @@ -543,6 +540,7 @@ LEAN_EXPORT lean_object* l_Lean_Server_ModuleRefs_toLspModuleRefs___boxed(lean_o LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Server_combineIdents_useConstRepresentatives___spec__10(lean_object*, lean_object*, lean_object*); size_t lean_usize_land(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Server_combineIdents(lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___closed__1; lean_object* l_Array_get_x3f___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Server_dedupReferences___closed__5; static lean_object* _init_l_Lean_Server_RefInfo_empty___closed__1() { @@ -10832,7 +10830,7 @@ x_29 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_29, 0, x_8); lean_ctor_set(x_29, 1, x_28); x_30 = l_Lean_Server_RefInfo_empty___closed__1; -x_31 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_29, x_30); +x_31 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_29, x_30); x_32 = l_Lean_Json_mkObj(x_31); return x_32; } @@ -10864,7 +10862,7 @@ x_41 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_41, 0, x_8); lean_ctor_set(x_41, 1, x_40); x_42 = l_Lean_Server_RefInfo_empty___closed__1; -x_43 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_41, x_42); +x_43 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_41, x_42); x_44 = l_Lean_Json_mkObj(x_43); return x_44; } @@ -10895,7 +10893,7 @@ x_55 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_55, 0, x_8); lean_ctor_set(x_55, 1, x_54); x_56 = l_Lean_Server_RefInfo_empty___closed__1; -x_57 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_55, x_56); +x_57 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_55, x_56); x_58 = l_Lean_Json_mkObj(x_57); return x_58; } @@ -11596,7 +11594,7 @@ return x_130; } } } -static lean_object* _init_l_panic___at_Lean_Server_findReferences___spec__4___closed__1() { +static lean_object* _init_l_panic___at_Lean_Server_findReferences___spec__3___closed__1() { _start: { lean_object* x_1; lean_object* x_2; @@ -11605,27 +11603,27 @@ x_2 = l_StateT_instMonad___rarg(x_1); return x_2; } } -static lean_object* _init_l_panic___at_Lean_Server_findReferences___spec__4___closed__2() { +static lean_object* _init_l_panic___at_Lean_Server_findReferences___spec__3___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_panic___at_Lean_Server_findReferences___spec__4___closed__1; +x_2 = l_panic___at_Lean_Server_findReferences___spec__3___closed__1; x_3 = l_instInhabitedOfMonad___rarg(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_panic___at_Lean_Server_findReferences___spec__4(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_panic___at_Lean_Server_findReferences___spec__3(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_3 = l_panic___at_Lean_Server_findReferences___spec__4___closed__2; +x_3 = l_panic___at_Lean_Server_findReferences___spec__3___closed__2; x_4 = lean_panic_fn(x_3, x_1); x_5 = lean_apply_1(x_4, x_2); return x_5; } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Server_findReferences___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Server_findReferences___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { if (lean_obj_tag(x_4) == 0) @@ -11652,7 +11650,7 @@ x_11 = lean_ctor_get(x_4, 1); lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_12 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3(x_1, x_2, x_3, x_10, x_6); +x_12 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2(x_1, x_2, x_3, x_10, x_6); x_13 = lean_ctor_get(x_12, 0); lean_inc(x_13); x_14 = lean_ctor_get(x_12, 1); @@ -11681,7 +11679,7 @@ lean_dec(x_4); lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_18 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3(x_1, x_2, x_3, x_16, x_6); +x_18 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2(x_1, x_2, x_3, x_16, x_6); x_19 = lean_ctor_get(x_18, 0); lean_inc(x_19); x_20 = lean_ctor_get(x_18, 1); @@ -11698,7 +11696,7 @@ goto _start; } } } -static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__1() { +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__1() { _start: { lean_object* x_1; @@ -11706,7 +11704,7 @@ x_1 = lean_mk_string_unchecked("Lean.Server.InfoUtils", 21, 21); return x_1; } } -static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__2() { +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__2() { _start: { lean_object* x_1; @@ -11714,7 +11712,7 @@ x_1 = lean_mk_string_unchecked("Lean.Elab.InfoTree.visitM.go", 28, 28); return x_1; } } -static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__3() { +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__3() { _start: { lean_object* x_1; @@ -11722,20 +11720,20 @@ x_1 = lean_mk_string_unchecked("unexpected context-free info tree node", 38, 38) return x_1; } } -static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__4() { +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__1; -x_2 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__2; -x_3 = lean_unsigned_to_nat(56u); +x_1 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__1; +x_2 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__2; +x_3 = lean_unsigned_to_nat(62u); x_4 = lean_unsigned_to_nat(21u); -x_5 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__3; +x_5 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { if (lean_obj_tag(x_3) == 0) @@ -11760,8 +11758,8 @@ lean_object* x_10; lean_object* x_11; lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_10 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__4; -x_11 = l_panic___at_Lean_Server_findReferences___spec__4(x_10, x_5); +x_10 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__4; +x_11 = l_panic___at_Lean_Server_findReferences___spec__3(x_10, x_5); return x_11; } default: @@ -11800,7 +11798,7 @@ uint8_t x_18; x_18 = !lean_is_exclusive(x_3); if (x_18 == 0) { -lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; x_19 = lean_ctor_get(x_3, 0); x_20 = lean_ctor_get(x_4, 0); lean_inc(x_20); @@ -11812,128 +11810,200 @@ lean_inc(x_21); lean_inc(x_20); lean_inc(x_19); x_22 = lean_apply_4(x_1, x_19, x_20, x_21, x_5); -x_23 = lean_ctor_get(x_22, 1); +x_23 = lean_ctor_get(x_22, 0); lean_inc(x_23); +x_24 = lean_unbox(x_23); +lean_dec(x_23); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; +lean_dec(x_1); +x_25 = lean_ctor_get(x_22, 1); +lean_inc(x_25); lean_dec(x_22); -lean_inc(x_19); -x_24 = l_Lean_Elab_Info_updateContext_x3f(x_3, x_20); -x_25 = l_Lean_PersistentArray_toList___rarg(x_21); x_26 = lean_box(0); -lean_inc(x_2); -x_27 = l_List_mapM_loop___at_Lean_Server_findReferences___spec__5(x_1, x_2, x_24, x_25, x_26, x_23); -x_28 = lean_ctor_get(x_27, 0); -lean_inc(x_28); -x_29 = lean_ctor_get(x_27, 1); -lean_inc(x_29); -lean_dec(x_27); -x_30 = lean_apply_5(x_2, x_19, x_20, x_21, x_28, x_29); -x_31 = !lean_is_exclusive(x_30); -if (x_31 == 0) +x_27 = lean_apply_5(x_2, x_19, x_20, x_21, x_26, x_25); +x_28 = !lean_is_exclusive(x_27); +if (x_28 == 0) { -lean_object* x_32; lean_object* x_33; -x_32 = lean_ctor_get(x_30, 0); -x_33 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_33, 0, x_32); -lean_ctor_set(x_30, 0, x_33); -return x_30; +lean_object* x_29; +x_29 = lean_ctor_get(x_27, 0); +lean_ctor_set(x_3, 0, x_29); +lean_ctor_set(x_27, 0, x_3); +return x_27; } else { -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_34 = lean_ctor_get(x_30, 0); -x_35 = lean_ctor_get(x_30, 1); -lean_inc(x_35); -lean_inc(x_34); -lean_dec(x_30); -x_36 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_36, 0, x_34); -x_37 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_37, 0, x_36); -lean_ctor_set(x_37, 1, x_35); -return x_37; +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_27, 0); +x_31 = lean_ctor_get(x_27, 1); +lean_inc(x_31); +lean_inc(x_30); +lean_dec(x_27); +lean_ctor_set(x_3, 0, x_30); +x_32 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_32, 0, x_3); +lean_ctor_set(x_32, 1, x_31); +return x_32; } } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_38 = lean_ctor_get(x_3, 0); +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; +x_33 = lean_ctor_get(x_22, 1); +lean_inc(x_33); +lean_dec(x_22); +lean_inc(x_19); +x_34 = l_Lean_Elab_Info_updateContext_x3f(x_3, x_20); +x_35 = l_Lean_PersistentArray_toList___rarg(x_21); +x_36 = lean_box(0); +lean_inc(x_2); +x_37 = l_List_mapM_loop___at_Lean_Server_findReferences___spec__4(x_1, x_2, x_34, x_35, x_36, x_33); +x_38 = lean_ctor_get(x_37, 0); lean_inc(x_38); -lean_dec(x_3); -x_39 = lean_ctor_get(x_4, 0); -lean_inc(x_39); -x_40 = lean_ctor_get(x_4, 1); -lean_inc(x_40); -lean_dec(x_4); -lean_inc(x_1); -lean_inc(x_40); +x_39 = lean_ctor_get(x_37, 1); lean_inc(x_39); -lean_inc(x_38); -x_41 = lean_apply_4(x_1, x_38, x_39, x_40, x_5); -x_42 = lean_ctor_get(x_41, 1); -lean_inc(x_42); -lean_dec(x_41); -lean_inc(x_38); +lean_dec(x_37); +x_40 = lean_apply_5(x_2, x_19, x_20, x_21, x_38, x_39); +x_41 = !lean_is_exclusive(x_40); +if (x_41 == 0) +{ +lean_object* x_42; lean_object* x_43; +x_42 = lean_ctor_get(x_40, 0); x_43 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_43, 0, x_38); -x_44 = l_Lean_Elab_Info_updateContext_x3f(x_43, x_39); -x_45 = l_Lean_PersistentArray_toList___rarg(x_40); -x_46 = lean_box(0); -lean_inc(x_2); -x_47 = l_List_mapM_loop___at_Lean_Server_findReferences___spec__5(x_1, x_2, x_44, x_45, x_46, x_42); -x_48 = lean_ctor_get(x_47, 0); +lean_ctor_set(x_43, 0, x_42); +lean_ctor_set(x_40, 0, x_43); +return x_40; +} +else +{ +lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_44 = lean_ctor_get(x_40, 0); +x_45 = lean_ctor_get(x_40, 1); +lean_inc(x_45); +lean_inc(x_44); +lean_dec(x_40); +x_46 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_46, 0, x_44); +x_47 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_47, 0, x_46); +lean_ctor_set(x_47, 1, x_45); +return x_47; +} +} +} +else +{ +lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; uint8_t x_53; +x_48 = lean_ctor_get(x_3, 0); lean_inc(x_48); -x_49 = lean_ctor_get(x_47, 1); +lean_dec(x_3); +x_49 = lean_ctor_get(x_4, 0); lean_inc(x_49); -lean_dec(x_47); -x_50 = lean_apply_5(x_2, x_38, x_39, x_40, x_48, x_49); -x_51 = lean_ctor_get(x_50, 0); -lean_inc(x_51); -x_52 = lean_ctor_get(x_50, 1); +x_50 = lean_ctor_get(x_4, 1); +lean_inc(x_50); +lean_dec(x_4); +lean_inc(x_1); +lean_inc(x_50); +lean_inc(x_49); +lean_inc(x_48); +x_51 = lean_apply_4(x_1, x_48, x_49, x_50, x_5); +x_52 = lean_ctor_get(x_51, 0); lean_inc(x_52); -if (lean_is_exclusive(x_50)) { - lean_ctor_release(x_50, 0); - lean_ctor_release(x_50, 1); - x_53 = x_50; +x_53 = lean_unbox(x_52); +lean_dec(x_52); +if (x_53 == 0) +{ +lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; +lean_dec(x_1); +x_54 = lean_ctor_get(x_51, 1); +lean_inc(x_54); +lean_dec(x_51); +x_55 = lean_box(0); +x_56 = lean_apply_5(x_2, x_48, x_49, x_50, x_55, x_54); +x_57 = lean_ctor_get(x_56, 0); +lean_inc(x_57); +x_58 = lean_ctor_get(x_56, 1); +lean_inc(x_58); +if (lean_is_exclusive(x_56)) { + lean_ctor_release(x_56, 0); + lean_ctor_release(x_56, 1); + x_59 = x_56; } else { - lean_dec_ref(x_50); - x_53 = lean_box(0); + lean_dec_ref(x_56); + x_59 = lean_box(0); } -x_54 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_54, 0, x_51); -if (lean_is_scalar(x_53)) { - x_55 = lean_alloc_ctor(0, 2, 0); +x_60 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_60, 0, x_57); +if (lean_is_scalar(x_59)) { + x_61 = lean_alloc_ctor(0, 2, 0); } else { - x_55 = x_53; + x_61 = x_59; +} +lean_ctor_set(x_61, 0, x_60); +lean_ctor_set(x_61, 1, x_58); +return x_61; +} +else +{ +lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; +x_62 = lean_ctor_get(x_51, 1); +lean_inc(x_62); +lean_dec(x_51); +lean_inc(x_48); +x_63 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_63, 0, x_48); +x_64 = l_Lean_Elab_Info_updateContext_x3f(x_63, x_49); +x_65 = l_Lean_PersistentArray_toList___rarg(x_50); +x_66 = lean_box(0); +lean_inc(x_2); +x_67 = l_List_mapM_loop___at_Lean_Server_findReferences___spec__4(x_1, x_2, x_64, x_65, x_66, x_62); +x_68 = lean_ctor_get(x_67, 0); +lean_inc(x_68); +x_69 = lean_ctor_get(x_67, 1); +lean_inc(x_69); +lean_dec(x_67); +x_70 = lean_apply_5(x_2, x_48, x_49, x_50, x_68, x_69); +x_71 = lean_ctor_get(x_70, 0); +lean_inc(x_71); +x_72 = lean_ctor_get(x_70, 1); +lean_inc(x_72); +if (lean_is_exclusive(x_70)) { + lean_ctor_release(x_70, 0); + lean_ctor_release(x_70, 1); + x_73 = x_70; +} else { + lean_dec_ref(x_70); + x_73 = lean_box(0); +} +x_74 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_74, 0, x_71); +if (lean_is_scalar(x_73)) { + x_75 = lean_alloc_ctor(0, 2, 0); +} else { + x_75 = x_73; +} +lean_ctor_set(x_75, 0, x_74); +lean_ctor_set(x_75, 1, x_72); +return x_75; } -lean_ctor_set(x_55, 0, x_54); -lean_ctor_set(x_55, 1, x_52); -return x_55; } } default: { -lean_object* x_56; lean_object* x_57; +lean_object* x_76; lean_object* x_77; lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_56 = lean_box(0); -x_57 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_57, 0, x_56); -lean_ctor_set(x_57, 1, x_5); -return x_57; -} -} +x_76 = lean_box(0); +x_77 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_77, 0, x_76); +lean_ctor_set(x_77, 1, x_5); +return x_77; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Server_findReferences___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -lean_object* x_5; lean_object* x_6; -x_5 = lean_box(0); -x_6 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3(x_1, x_2, x_5, x_3, x_4); -return x_6; } } LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_findReferences___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { @@ -11944,49 +12014,50 @@ x_7 = lean_apply_4(x_1, x_2, x_3, x_4, x_6); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_findReferences___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_findReferences___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_5; lean_object* x_6; uint8_t x_7; -x_5 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_findReferences___spec__1___lambda__1___boxed), 6, 1); -lean_closure_set(x_5, 0, x_2); -x_6 = l_Lean_Elab_InfoTree_visitM___at_Lean_Server_findReferences___spec__2(x_1, x_5, x_3, x_4); -x_7 = !lean_is_exclusive(x_6); -if (x_7 == 0) +lean_object* x_6; lean_object* x_7; uint8_t x_8; +x_6 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_findReferences___spec__1___lambda__1___boxed), 6, 1); +lean_closure_set(x_6, 0, x_2); +x_7 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2(x_1, x_6, x_3, x_4, x_5); +x_8 = !lean_is_exclusive(x_7); +if (x_8 == 0) { -lean_object* x_8; lean_object* x_9; -x_8 = lean_ctor_get(x_6, 0); -lean_dec(x_8); -x_9 = lean_box(0); -lean_ctor_set(x_6, 0, x_9); -return x_6; +lean_object* x_9; lean_object* x_10; +x_9 = lean_ctor_get(x_7, 0); +lean_dec(x_9); +x_10 = lean_box(0); +lean_ctor_set(x_7, 0, x_10); +return x_7; } else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_10 = lean_ctor_get(x_6, 1); -lean_inc(x_10); -lean_dec(x_6); -x_11 = lean_box(0); -x_12 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_12, 0, x_11); -lean_ctor_set(x_12, 1, x_10); -return x_12; +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_7, 1); +lean_inc(x_11); +lean_dec(x_7); +x_12 = lean_box(0); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_11); +return x_13; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_5; lean_object* x_6; -x_5 = lean_box(0); -x_6 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_6, 0, x_5); -lean_ctor_set(x_6, 1, x_4); -return x_6; +uint8_t x_5; lean_object* x_6; lean_object* x_7; +x_5 = 1; +x_6 = lean_box(x_5); +x_7 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_7, 0, x_6); +lean_ctor_set(x_7, 1, x_4); +return x_7; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; @@ -12157,15 +12228,15 @@ return x_41; } } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___closed__1() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___lambda__1___boxed), 4, 0); +x_1 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___lambda__1___boxed), 4, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6) { _start: { uint8_t x_7; @@ -12181,23 +12252,24 @@ return x_8; } else { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; size_t x_14; size_t x_15; lean_object* x_16; +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; size_t x_15; size_t x_16; lean_object* x_17; lean_dec(x_5); x_9 = lean_array_uget(x_2, x_4); lean_inc(x_1); -x_10 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___lambda__2___boxed), 5, 1); +x_10 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___lambda__2___boxed), 5, 1); lean_closure_set(x_10, 0, x_1); -x_11 = l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___closed__1; -x_12 = l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_findReferences___spec__1(x_11, x_10, x_9, x_6); -x_13 = lean_ctor_get(x_12, 1); -lean_inc(x_13); -lean_dec(x_12); -x_14 = 1; -x_15 = lean_usize_add(x_4, x_14); -x_16 = lean_box(0); -x_4 = x_15; -x_5 = x_16; -x_6 = x_13; +x_11 = lean_box(0); +x_12 = l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___closed__1; +x_13 = l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_findReferences___spec__1(x_12, x_10, x_11, x_9, x_6); +x_14 = lean_ctor_get(x_13, 1); +lean_inc(x_14); +lean_dec(x_13); +x_15 = 1; +x_16 = lean_usize_add(x_4, x_15); +x_17 = lean_box(0); +x_4 = x_16; +x_5 = x_17; +x_6 = x_14; goto _start; } } @@ -12210,7 +12282,7 @@ x_3 = lean_array_size(x_2); x_4 = 0; x_5 = lean_box(0); x_6 = l_Lean_Server_RefInfo_empty___closed__1; -x_7 = l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5(x_1, x_2, x_3, x_4, x_5, x_6); x_8 = lean_ctor_get(x_7, 1); lean_inc(x_8); lean_dec(x_7); @@ -12226,27 +12298,27 @@ lean_dec(x_5); return x_7; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___lambda__1(x_1, x_2, x_3, x_4); +x_5 = l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___lambda__1(x_1, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); return x_5; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; -x_6 = l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___lambda__2(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___lambda__2(x_1, x_2, x_3, x_4, x_5); lean_dec(x_4); return x_6; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { size_t x_7; size_t x_8; lean_object* x_9; @@ -12254,7 +12326,7 @@ x_7 = lean_unbox_usize(x_3); lean_dec(x_3); x_8 = lean_unbox_usize(x_4); lean_dec(x_4); -x_9 = l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6(x_1, x_2, x_7, x_8, x_5, x_6); +x_9 = l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5(x_1, x_2, x_7, x_8, x_5, x_6); lean_dec(x_2); return x_9; } @@ -15523,17 +15595,17 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_panic___at_Lean_Server_combineIdents_buildIdMap___spec__6(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_panic___at_Lean_Server_combineIdents_buildIdMap___spec__5(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_3 = l_panic___at_Lean_Server_findReferences___spec__4___closed__2; +x_3 = l_panic___at_Lean_Server_findReferences___spec__3___closed__2; x_4 = lean_panic_fn(x_3, x_1); x_5 = lean_apply_1(x_4, x_2); return x_5; } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Server_combineIdents_buildIdMap___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Server_combineIdents_buildIdMap___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { if (lean_obj_tag(x_4) == 0) @@ -15560,7 +15632,7 @@ x_11 = lean_ctor_get(x_4, 1); lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_12 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_combineIdents_buildIdMap___spec__5(x_1, x_2, x_3, x_10, x_6); +x_12 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_combineIdents_buildIdMap___spec__4(x_1, x_2, x_3, x_10, x_6); x_13 = lean_ctor_get(x_12, 0); lean_inc(x_13); x_14 = lean_ctor_get(x_12, 1); @@ -15589,7 +15661,7 @@ lean_dec(x_4); lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_18 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_combineIdents_buildIdMap___spec__5(x_1, x_2, x_3, x_16, x_6); +x_18 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_combineIdents_buildIdMap___spec__4(x_1, x_2, x_3, x_16, x_6); x_19 = lean_ctor_get(x_18, 0); lean_inc(x_19); x_20 = lean_ctor_get(x_18, 1); @@ -15606,7 +15678,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_combineIdents_buildIdMap___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_combineIdents_buildIdMap___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { if (lean_obj_tag(x_3) == 0) @@ -15631,8 +15703,8 @@ lean_object* x_10; lean_object* x_11; lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_10 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__4; -x_11 = l_panic___at_Lean_Server_combineIdents_buildIdMap___spec__6(x_10, x_5); +x_10 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__4; +x_11 = l_panic___at_Lean_Server_combineIdents_buildIdMap___spec__5(x_10, x_5); return x_11; } default: @@ -15671,7 +15743,7 @@ uint8_t x_18; x_18 = !lean_is_exclusive(x_3); if (x_18 == 0) { -lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; x_19 = lean_ctor_get(x_3, 0); x_20 = lean_ctor_get(x_4, 0); lean_inc(x_20); @@ -15683,162 +15755,234 @@ lean_inc(x_21); lean_inc(x_20); lean_inc(x_19); x_22 = lean_apply_4(x_1, x_19, x_20, x_21, x_5); -x_23 = lean_ctor_get(x_22, 1); +x_23 = lean_ctor_get(x_22, 0); lean_inc(x_23); +x_24 = lean_unbox(x_23); +lean_dec(x_23); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; +lean_dec(x_1); +x_25 = lean_ctor_get(x_22, 1); +lean_inc(x_25); lean_dec(x_22); -lean_inc(x_19); -x_24 = l_Lean_Elab_Info_updateContext_x3f(x_3, x_20); -x_25 = l_Lean_PersistentArray_toList___rarg(x_21); x_26 = lean_box(0); -lean_inc(x_2); -x_27 = l_List_mapM_loop___at_Lean_Server_combineIdents_buildIdMap___spec__7(x_1, x_2, x_24, x_25, x_26, x_23); -x_28 = lean_ctor_get(x_27, 0); -lean_inc(x_28); -x_29 = lean_ctor_get(x_27, 1); -lean_inc(x_29); -lean_dec(x_27); -x_30 = lean_apply_5(x_2, x_19, x_20, x_21, x_28, x_29); -x_31 = !lean_is_exclusive(x_30); -if (x_31 == 0) +x_27 = lean_apply_5(x_2, x_19, x_20, x_21, x_26, x_25); +x_28 = !lean_is_exclusive(x_27); +if (x_28 == 0) { -lean_object* x_32; lean_object* x_33; -x_32 = lean_ctor_get(x_30, 0); -x_33 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_33, 0, x_32); -lean_ctor_set(x_30, 0, x_33); -return x_30; +lean_object* x_29; +x_29 = lean_ctor_get(x_27, 0); +lean_ctor_set(x_3, 0, x_29); +lean_ctor_set(x_27, 0, x_3); +return x_27; } else { -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_34 = lean_ctor_get(x_30, 0); -x_35 = lean_ctor_get(x_30, 1); -lean_inc(x_35); -lean_inc(x_34); -lean_dec(x_30); -x_36 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_36, 0, x_34); -x_37 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_37, 0, x_36); -lean_ctor_set(x_37, 1, x_35); -return x_37; +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_27, 0); +x_31 = lean_ctor_get(x_27, 1); +lean_inc(x_31); +lean_inc(x_30); +lean_dec(x_27); +lean_ctor_set(x_3, 0, x_30); +x_32 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_32, 0, x_3); +lean_ctor_set(x_32, 1, x_31); +return x_32; } } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_38 = lean_ctor_get(x_3, 0); +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; +x_33 = lean_ctor_get(x_22, 1); +lean_inc(x_33); +lean_dec(x_22); +lean_inc(x_19); +x_34 = l_Lean_Elab_Info_updateContext_x3f(x_3, x_20); +x_35 = l_Lean_PersistentArray_toList___rarg(x_21); +x_36 = lean_box(0); +lean_inc(x_2); +x_37 = l_List_mapM_loop___at_Lean_Server_combineIdents_buildIdMap___spec__6(x_1, x_2, x_34, x_35, x_36, x_33); +x_38 = lean_ctor_get(x_37, 0); lean_inc(x_38); -lean_dec(x_3); -x_39 = lean_ctor_get(x_4, 0); -lean_inc(x_39); -x_40 = lean_ctor_get(x_4, 1); -lean_inc(x_40); -lean_dec(x_4); -lean_inc(x_1); -lean_inc(x_40); +x_39 = lean_ctor_get(x_37, 1); lean_inc(x_39); -lean_inc(x_38); -x_41 = lean_apply_4(x_1, x_38, x_39, x_40, x_5); -x_42 = lean_ctor_get(x_41, 1); -lean_inc(x_42); -lean_dec(x_41); -lean_inc(x_38); +lean_dec(x_37); +x_40 = lean_apply_5(x_2, x_19, x_20, x_21, x_38, x_39); +x_41 = !lean_is_exclusive(x_40); +if (x_41 == 0) +{ +lean_object* x_42; lean_object* x_43; +x_42 = lean_ctor_get(x_40, 0); x_43 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_43, 0, x_38); -x_44 = l_Lean_Elab_Info_updateContext_x3f(x_43, x_39); -x_45 = l_Lean_PersistentArray_toList___rarg(x_40); -x_46 = lean_box(0); -lean_inc(x_2); -x_47 = l_List_mapM_loop___at_Lean_Server_combineIdents_buildIdMap___spec__7(x_1, x_2, x_44, x_45, x_46, x_42); -x_48 = lean_ctor_get(x_47, 0); +lean_ctor_set(x_43, 0, x_42); +lean_ctor_set(x_40, 0, x_43); +return x_40; +} +else +{ +lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_44 = lean_ctor_get(x_40, 0); +x_45 = lean_ctor_get(x_40, 1); +lean_inc(x_45); +lean_inc(x_44); +lean_dec(x_40); +x_46 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_46, 0, x_44); +x_47 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_47, 0, x_46); +lean_ctor_set(x_47, 1, x_45); +return x_47; +} +} +} +else +{ +lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; uint8_t x_53; +x_48 = lean_ctor_get(x_3, 0); lean_inc(x_48); -x_49 = lean_ctor_get(x_47, 1); +lean_dec(x_3); +x_49 = lean_ctor_get(x_4, 0); lean_inc(x_49); -lean_dec(x_47); -x_50 = lean_apply_5(x_2, x_38, x_39, x_40, x_48, x_49); -x_51 = lean_ctor_get(x_50, 0); -lean_inc(x_51); -x_52 = lean_ctor_get(x_50, 1); +x_50 = lean_ctor_get(x_4, 1); +lean_inc(x_50); +lean_dec(x_4); +lean_inc(x_1); +lean_inc(x_50); +lean_inc(x_49); +lean_inc(x_48); +x_51 = lean_apply_4(x_1, x_48, x_49, x_50, x_5); +x_52 = lean_ctor_get(x_51, 0); lean_inc(x_52); -if (lean_is_exclusive(x_50)) { - lean_ctor_release(x_50, 0); - lean_ctor_release(x_50, 1); - x_53 = x_50; +x_53 = lean_unbox(x_52); +lean_dec(x_52); +if (x_53 == 0) +{ +lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; +lean_dec(x_1); +x_54 = lean_ctor_get(x_51, 1); +lean_inc(x_54); +lean_dec(x_51); +x_55 = lean_box(0); +x_56 = lean_apply_5(x_2, x_48, x_49, x_50, x_55, x_54); +x_57 = lean_ctor_get(x_56, 0); +lean_inc(x_57); +x_58 = lean_ctor_get(x_56, 1); +lean_inc(x_58); +if (lean_is_exclusive(x_56)) { + lean_ctor_release(x_56, 0); + lean_ctor_release(x_56, 1); + x_59 = x_56; } else { - lean_dec_ref(x_50); - x_53 = lean_box(0); + lean_dec_ref(x_56); + x_59 = lean_box(0); } -x_54 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_54, 0, x_51); -if (lean_is_scalar(x_53)) { - x_55 = lean_alloc_ctor(0, 2, 0); +x_60 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_60, 0, x_57); +if (lean_is_scalar(x_59)) { + x_61 = lean_alloc_ctor(0, 2, 0); } else { - x_55 = x_53; + x_61 = x_59; +} +lean_ctor_set(x_61, 0, x_60); +lean_ctor_set(x_61, 1, x_58); +return x_61; +} +else +{ +lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; +x_62 = lean_ctor_get(x_51, 1); +lean_inc(x_62); +lean_dec(x_51); +lean_inc(x_48); +x_63 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_63, 0, x_48); +x_64 = l_Lean_Elab_Info_updateContext_x3f(x_63, x_49); +x_65 = l_Lean_PersistentArray_toList___rarg(x_50); +x_66 = lean_box(0); +lean_inc(x_2); +x_67 = l_List_mapM_loop___at_Lean_Server_combineIdents_buildIdMap___spec__6(x_1, x_2, x_64, x_65, x_66, x_62); +x_68 = lean_ctor_get(x_67, 0); +lean_inc(x_68); +x_69 = lean_ctor_get(x_67, 1); +lean_inc(x_69); +lean_dec(x_67); +x_70 = lean_apply_5(x_2, x_48, x_49, x_50, x_68, x_69); +x_71 = lean_ctor_get(x_70, 0); +lean_inc(x_71); +x_72 = lean_ctor_get(x_70, 1); +lean_inc(x_72); +if (lean_is_exclusive(x_70)) { + lean_ctor_release(x_70, 0); + lean_ctor_release(x_70, 1); + x_73 = x_70; +} else { + lean_dec_ref(x_70); + x_73 = lean_box(0); +} +x_74 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_74, 0, x_71); +if (lean_is_scalar(x_73)) { + x_75 = lean_alloc_ctor(0, 2, 0); +} else { + x_75 = x_73; +} +lean_ctor_set(x_75, 0, x_74); +lean_ctor_set(x_75, 1, x_72); +return x_75; } -lean_ctor_set(x_55, 0, x_54); -lean_ctor_set(x_55, 1, x_52); -return x_55; } } default: { -lean_object* x_56; lean_object* x_57; +lean_object* x_76; lean_object* x_77; lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_56 = lean_box(0); -x_57 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_57, 0, x_56); -lean_ctor_set(x_57, 1, x_5); -return x_57; -} +x_76 = lean_box(0); +x_77 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_77, 0, x_76); +lean_ctor_set(x_77, 1, x_5); +return x_77; } } } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Server_combineIdents_buildIdMap___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -lean_object* x_5; lean_object* x_6; -x_5 = lean_box(0); -x_6 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_combineIdents_buildIdMap___spec__5(x_1, x_2, x_5, x_3, x_4); -return x_6; -} } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_combineIdents_buildIdMap___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_combineIdents_buildIdMap___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_5; lean_object* x_6; uint8_t x_7; -x_5 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_findReferences___spec__1___lambda__1___boxed), 6, 1); -lean_closure_set(x_5, 0, x_2); -x_6 = l_Lean_Elab_InfoTree_visitM___at_Lean_Server_combineIdents_buildIdMap___spec__4(x_1, x_5, x_3, x_4); -x_7 = !lean_is_exclusive(x_6); -if (x_7 == 0) +lean_object* x_6; lean_object* x_7; uint8_t x_8; +x_6 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_findReferences___spec__1___lambda__1___boxed), 6, 1); +lean_closure_set(x_6, 0, x_2); +x_7 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_combineIdents_buildIdMap___spec__4(x_1, x_6, x_3, x_4, x_5); +x_8 = !lean_is_exclusive(x_7); +if (x_8 == 0) { -lean_object* x_8; lean_object* x_9; -x_8 = lean_ctor_get(x_6, 0); -lean_dec(x_8); -x_9 = lean_box(0); -lean_ctor_set(x_6, 0, x_9); -return x_6; +lean_object* x_9; lean_object* x_10; +x_9 = lean_ctor_get(x_7, 0); +lean_dec(x_9); +x_10 = lean_box(0); +lean_ctor_set(x_7, 0, x_10); +return x_7; } else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_10 = lean_ctor_get(x_6, 1); -lean_inc(x_10); -lean_dec(x_6); -x_11 = lean_box(0); -x_12 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_12, 0, x_11); -lean_ctor_set(x_12, 1, x_10); -return x_12; +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_7, 1); +lean_inc(x_11); +lean_dec(x_7); +x_12 = lean_box(0); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_11); +return x_13; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__7___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { if (lean_obj_tag(x_2) == 9) @@ -15892,46 +16036,47 @@ return x_21; } } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8___closed__1() { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__7___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8___lambda__1___boxed), 4, 0); +x_1 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__7___lambda__1___boxed), 4, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__7(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5) { _start: { uint8_t x_6; x_6 = lean_usize_dec_eq(x_2, x_3); if (x_6 == 0) { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; size_t x_13; size_t x_14; +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; size_t x_14; size_t x_15; lean_dec(x_4); x_7 = lean_array_uget(x_1, x_2); -x_8 = l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___closed__1; -x_9 = l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8___closed__1; -x_10 = l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_combineIdents_buildIdMap___spec__3(x_8, x_9, x_7, x_5); -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -x_12 = lean_ctor_get(x_10, 1); +x_8 = lean_box(0); +x_9 = l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___closed__1; +x_10 = l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__7___closed__1; +x_11 = l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_combineIdents_buildIdMap___spec__3(x_9, x_10, x_8, x_7, x_5); +x_12 = lean_ctor_get(x_11, 0); lean_inc(x_12); -lean_dec(x_10); -x_13 = 1; -x_14 = lean_usize_add(x_2, x_13); -x_2 = x_14; -x_4 = x_11; -x_5 = x_12; +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +x_14 = 1; +x_15 = lean_usize_add(x_2, x_14); +x_2 = x_15; +x_4 = x_12; +x_5 = x_13; goto _start; } else { -lean_object* x_16; -x_16 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_16, 0, x_4); -lean_ctor_set(x_16, 1, x_5); -return x_16; +lean_object* x_17; +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_4); +lean_ctor_set(x_17, 1, x_5); +return x_17; } } } @@ -15969,7 +16114,7 @@ else size_t x_14; lean_object* x_15; lean_object* x_16; x_14 = lean_usize_of_nat(x_10); lean_dec(x_10); -x_15 = l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8(x_1, x_5, x_14, x_6, x_9); +x_15 = l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__7(x_1, x_5, x_14, x_6, x_9); x_16 = lean_ctor_get(x_15, 1); lean_inc(x_16); lean_dec(x_15); @@ -16002,16 +16147,16 @@ lean_dec(x_1); return x_9; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__7___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8___lambda__1(x_1, x_2, x_3, x_4); +x_5 = l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__7___lambda__1(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { size_t x_6; size_t x_7; lean_object* x_8; @@ -16019,7 +16164,7 @@ x_6 = lean_unbox_usize(x_2); lean_dec(x_2); x_7 = lean_unbox_usize(x_3); lean_dec(x_3); -x_8 = l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8(x_1, x_6, x_7, x_4, x_5); +x_8 = l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__7(x_1, x_6, x_7, x_4, x_5); lean_dec(x_1); return x_8; } @@ -28052,22 +28197,22 @@ l_Lean_Server_Ilean_load___closed__2 = _init_l_Lean_Server_Ilean_load___closed__ lean_mark_persistent(l_Lean_Server_Ilean_load___closed__2); l_Lean_Server_Ilean_load___closed__3 = _init_l_Lean_Server_Ilean_load___closed__3(); lean_mark_persistent(l_Lean_Server_Ilean_load___closed__3); -l_panic___at_Lean_Server_findReferences___spec__4___closed__1 = _init_l_panic___at_Lean_Server_findReferences___spec__4___closed__1(); -lean_mark_persistent(l_panic___at_Lean_Server_findReferences___spec__4___closed__1); -l_panic___at_Lean_Server_findReferences___spec__4___closed__2 = _init_l_panic___at_Lean_Server_findReferences___spec__4___closed__2(); -lean_mark_persistent(l_panic___at_Lean_Server_findReferences___spec__4___closed__2); -l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__1 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__1(); -lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__1); -l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__2 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__2(); -lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__2); -l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__3 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__3(); -lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__3); -l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__4 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__4(); -lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__4); -l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___closed__1); -l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8___closed__1 = _init_l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8___closed__1(); -lean_mark_persistent(l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8___closed__1); +l_panic___at_Lean_Server_findReferences___spec__3___closed__1 = _init_l_panic___at_Lean_Server_findReferences___spec__3___closed__1(); +lean_mark_persistent(l_panic___at_Lean_Server_findReferences___spec__3___closed__1); +l_panic___at_Lean_Server_findReferences___spec__3___closed__2 = _init_l_panic___at_Lean_Server_findReferences___spec__3___closed__2(); +lean_mark_persistent(l_panic___at_Lean_Server_findReferences___spec__3___closed__2); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__1 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__1(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__1); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__2 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__2(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__2); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__3 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__3(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__3); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__4 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__4(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__4); +l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___closed__1(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___closed__1); +l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__7___closed__1 = _init_l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__7___closed__1(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__7___closed__1); l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_dedupReferences___spec__4___at_Lean_Server_dedupReferences___spec__5___closed__1 = _init_l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_dedupReferences___spec__4___at_Lean_Server_dedupReferences___spec__5___closed__1(); l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_dedupReferences___spec__4___at_Lean_Server_dedupReferences___spec__5___closed__2 = _init_l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_dedupReferences___spec__4___at_Lean_Server_dedupReferences___spec__5___closed__2(); l_Array_qsort_sort___at_Lean_Server_dedupReferences___spec__10___closed__1 = _init_l_Array_qsort_sort___at_Lean_Server_dedupReferences___spec__10___closed__1(); diff --git a/stage0/stdlib/Lean/Server/Rpc/Basic.c b/stage0/stdlib/Lean/Server/Rpc/Basic.c index d514e6e87185..f56e0cceeaae 100644 --- a/stage0/stdlib/Lean/Server/Rpc/Basic.c +++ b/stage0/stdlib/Lean/Server/Rpc/Basic.c @@ -49,6 +49,7 @@ LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Server_rpc LEAN_EXPORT uint64_t l___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_hashRpcRef____x40_Lean_Server_Rpc_Basic___hyg_74_(size_t); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_Server_rpcGetRef___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_Server_instRpcEncodableOfFromJsonOfToJson___spec__1___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_Server_rpcGetRef___spec__1___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_fromJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_106____closed__2; static lean_object* l_Lean_Server_instRpcEncodableOption___rarg___lambda__2___closed__1; @@ -116,7 +117,6 @@ LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_erase___at_Lean_Server_rpcRele LEAN_EXPORT uint8_t l___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_beqRpcRef____x40_Lean_Server_Rpc_Basic___hyg_16_(size_t, size_t); static lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_fromJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_106____spec__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodableOfFromJsonOfToJson(lean_object*); -LEAN_EXPORT lean_object* l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_fromJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_106____closed__13; static lean_object* l_Lean_Lsp_instToJsonRpcRef___closed__1; static lean_object* l___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_fromJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_106____closed__5; @@ -592,7 +592,7 @@ x_1 = l_Lean_Lsp_instFromJsonRpcRef___closed__1; return x_1; } } -LEAN_EXPORT lean_object* l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -643,7 +643,7 @@ x_8 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_8, 0, x_7); lean_ctor_set(x_8, 1, x_6); x_9 = l___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____closed__1; -x_10 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_8, x_9); +x_10 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_8, x_9); x_11 = l_Lean_Json_mkObj(x_10); return x_11; } diff --git a/stage0/stdlib/Lean/Server/Rpc/Deriving.c b/stage0/stdlib/Lean/Server/Rpc/Deriving.c index 62fb45abd66c..d808cf4a50b5 100644 --- a/stage0/stdlib/Lean/Server/Rpc/Deriving.c +++ b/stage0/stdlib/Lean/Server/Rpc/Deriving.c @@ -18,6 +18,7 @@ static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncod lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__1___closed__12; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__89; +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__48; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__90; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___lambda__1___closed__9; @@ -29,13 +30,12 @@ static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncod LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___spec__10(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_RpcEncodable_deriveInductiveInstance___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___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___lambda__1___closed__39; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__4(size_t, size_t, lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); -static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__4; static lean_object* l_Lean_Server_RpcEncodable_isOptField___closed__1; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__1___closed__59; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__1___closed__34; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__21; +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___lambda__1___closed__33; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___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_RpcEncodable_deriveStructureInstance___closed__2; @@ -44,16 +44,19 @@ static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Derivi static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__1___closed__13; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__104; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___spec__8(size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__119; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__6___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___lambda__1___closed__14; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___spec__19(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__7(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_RpcEncodable_deriveStructureInstance___closed__1; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__68; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___closed__8; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__17; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__1___closed__19; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__66; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__6___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_toString(lean_object*, uint8_t, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__109; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___closed__7; @@ -63,7 +66,7 @@ static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncod static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__31; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__103; lean_object* l_Lean_MessageData_ofList(lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__2___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_RpcEncodable_deriveInstance___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___lambda__1___closed__26; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__38; @@ -71,15 +74,12 @@ static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncod static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__112; uint8_t lean_usize_dec_eq(size_t, size_t); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__1___closed__4; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3(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_RpcEncodable_deriveStructureInstance___spec__1___closed__51; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__19; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__91; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__1___closed__17; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__1___closed__53; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__4___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__121; -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___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___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__30; lean_object* l_Lean_Elab_Command_elabCommand(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); @@ -94,6 +94,7 @@ static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deri LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___spec__7(lean_object*, size_t, size_t, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__78; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__1___closed__27; +lean_object* lean_environment_find(lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__1___closed__5; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__61; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__32; @@ -148,17 +149,17 @@ LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeReducing___at___private_Lean size_t lean_usize_of_nat(lean_object*); static lean_object* l_Lean_Server_RpcEncodable_initFn____x40_Lean_Server_Rpc_Deriving___hyg_4847____closed__13; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__54; +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__4___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_RpcEncodable_deriveStructureInstance___spec__1___closed__9; static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___spec__11___closed__1; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__1___closed__60; -static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__5; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__35; static lean_object* l_Lean_Server_RpcEncodable_initFn____x40_Lean_Server_Rpc_Deriving___hyg_4847____closed__4; lean_object* l_Lean_Elab_registerDerivingHandler(lean_object*, lean_object*, lean_object*); uint8_t l_instDecidableNot___rarg(uint8_t); -lean_object* l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__37; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__43; +static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__3; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__1___closed__6; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___spec__5(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -174,6 +175,7 @@ static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncod lean_object* l_Lean_Meta_isType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___lambda__1___closed__12; static lean_object* l_Lean_Server_RpcEncodable_initFn____x40_Lean_Server_Rpc_Deriving___hyg_4847____closed__1; +static lean_object* l_Lean_getConstInfo___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__2___closed__1; lean_object* l_Lean_Syntax_node6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, 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_Server_RpcEncodable_isOptField___lambda__1___boxed(lean_object*); @@ -194,6 +196,7 @@ static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deri LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_matchAltTerm; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__58; lean_object* l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(lean_object*, lean_object*); +static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__6; static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___spec__14___lambda__1___closed__12; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___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*); lean_object* l_Lean_mkCIdentFrom(lean_object*, lean_object*, uint8_t); @@ -204,6 +207,7 @@ static lean_object* l_Lean_Server_RpcEncodable_isOptField___closed__3; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__9; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__2(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__1___closed__44; +static lean_object* l_Lean_getConstInfo___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__2___closed__2; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___lambda__1___closed__29; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__124; lean_object* l_Lean_Elab_Command_liftTermElabM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); @@ -219,6 +223,7 @@ static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncod static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__1___closed__8; lean_object* lean_array_to_list(lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__51; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5(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_getConstInfoCtor___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___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_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); @@ -233,7 +238,6 @@ static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncod static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__2; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__1___closed__31; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__22; -static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__1; LEAN_EXPORT lean_object* l_Lean_getConstInfoInduct___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__1___closed__30; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__47; @@ -301,17 +305,15 @@ static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncod LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); -lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__3___closed__7; lean_object* l_Lean_MessageData_ofExpr(lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__113; -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___lambda__1___closed__19; LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_RpcEncodable_initFn____x40_Lean_Server_Rpc_Deriving___hyg_4847____closed__15; static lean_object* l_Lean_getConstInfoInduct___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__1___closed__1; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__6(size_t, size_t, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__1___closed__16; -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_userName(lean_object*); lean_object* l_Lean_Syntax_node4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__1___closed__37; @@ -323,12 +325,12 @@ static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncod static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__99; LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___spec__13___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_RpcEncodable_initFn____x40_Lean_Server_Rpc_Deriving___hyg_4847____closed__12; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___spec__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__16; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__115; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__36; -static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__3; lean_object* lean_string_length(lean_object*); lean_object* l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); @@ -347,6 +349,7 @@ static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncod LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_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_RpcEncodable_deriveStructureInstance___lambda__1___closed__123; lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); +static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__4; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__105; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__95; LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -364,6 +367,7 @@ static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deri lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__63; static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__3___closed__2; +static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___spec__13(lean_object*); static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__3___closed__1; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__1___closed__29; @@ -375,6 +379,7 @@ uint8_t l_Lean_isStructure(lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__1___closed__41; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__8; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__1___closed__38; +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_RpcEncodable_instCoeTSyntaxConsSyntaxNodeKindStrNumAnonymousOfNatNatNilMkStr4___boxed(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__1___closed__39; static lean_object* l_Lean_getConstInfoInduct___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__1___closed__2; @@ -395,6 +400,7 @@ static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncod uint8_t l_Substring_beq(lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); static lean_object* l_Lean_Server_RpcEncodable_initFn____x40_Lean_Server_Rpc_Deriving___hyg_4847____closed__16; +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___closed__6; static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___spec__14___lambda__1___closed__6; static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___spec__4___closed__2; @@ -418,12 +424,12 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_D static lean_object* l_Lean_Server_RpcEncodable_initFn____x40_Lean_Server_Rpc_Deriving___hyg_4847____closed__5; static lean_object* l_Lean_Server_RpcEncodable_initFn____x40_Lean_Server_Rpc_Deriving___hyg_4847____closed__10; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__45; -static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__2; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__26; lean_object* l_Lean_Parser_Term_matchAlt(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___spec__18(size_t, size_t, lean_object*); lean_object* lean_array_get_size(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___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_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__5; LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__1___closed__47; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__77; @@ -436,8 +442,8 @@ static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncod static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__1___closed__24; uint8_t lean_usize_dec_lt(size_t, size_t); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__98; +lean_object* l_Lean_throwError___at_Lean_withSetOptionIn___spec__7(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__18; -static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__6; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___closed__3; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___lambda__1___closed__24; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__1___closed__21; @@ -457,11 +463,11 @@ static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncod static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___lambda__1___closed__32; lean_object* l_String_toSubstring_x27(lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__23; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___lambda__1___closed__38; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); lean_object* l_Lean_MessageData_ofName(lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___lambda__1___closed__27; +static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__2; 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*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__79; lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallTelescopeReducingImp___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -14680,7 +14686,204 @@ lean_dec(x_3); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___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___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_5 = l_Lean_Elab_Command_getRef(x_2, x_3, x_4); +x_6 = lean_ctor_get(x_5, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_5, 1); +lean_inc(x_7); +lean_dec(x_5); +x_8 = lean_ctor_get(x_2, 4); +lean_inc(x_8); +lean_inc(x_8); +x_9 = l_Lean_Elab_getBetterRef(x_6, x_8); +lean_dec(x_6); +x_10 = l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1(x_1, x_2, x_3, x_7); +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_12 = lean_ctor_get(x_10, 0); +x_13 = lean_ctor_get(x_10, 1); +x_14 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_12, x_8, x_2, x_3, x_13); +lean_dec(x_2); +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 0) +{ +lean_object* x_16; +x_16 = lean_ctor_get(x_14, 0); +lean_ctor_set(x_10, 1, x_16); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set_tag(x_14, 1); +lean_ctor_set(x_14, 0, x_10); +return x_14; +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_14, 0); +x_18 = lean_ctor_get(x_14, 1); +lean_inc(x_18); +lean_inc(x_17); +lean_dec(x_14); +lean_ctor_set(x_10, 1, x_17); +lean_ctor_set(x_10, 0, x_9); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_10); +lean_ctor_set(x_19, 1, 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; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_20 = lean_ctor_get(x_10, 0); +x_21 = lean_ctor_get(x_10, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_10); +x_22 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(x_20, x_8, x_2, x_3, x_21); +lean_dec(x_2); +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +if (lean_is_exclusive(x_22)) { + lean_ctor_release(x_22, 0); + lean_ctor_release(x_22, 1); + x_25 = x_22; +} else { + lean_dec_ref(x_22); + x_25 = lean_box(0); +} +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_9); +lean_ctor_set(x_26, 1, x_23); +if (lean_is_scalar(x_25)) { + x_27 = lean_alloc_ctor(1, 2, 0); +} else { + x_27 = x_25; + lean_ctor_set_tag(x_27, 1); +} +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_24); +return x_27; +} +} +} +static lean_object* _init_l_Lean_getConstInfo___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__2___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("unknown constant '", 18, 18); +return x_1; +} +} +static lean_object* _init_l_Lean_getConstInfo___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__2___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_getConstInfo___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__2___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; uint8_t x_6; +x_5 = lean_st_ref_get(x_3, x_4); +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; +x_7 = lean_ctor_get(x_5, 0); +x_8 = lean_ctor_get(x_5, 1); +x_9 = lean_ctor_get(x_7, 0); +lean_inc(x_9); +lean_dec(x_7); +lean_inc(x_1); +x_10 = lean_environment_find(x_9, x_1); +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; +lean_free_object(x_5); +x_11 = lean_box(0); +x_12 = l_Lean_Expr_const___override(x_1, x_11); +x_13 = l_Lean_MessageData_ofExpr(x_12); +x_14 = l_Lean_getConstInfo___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__2___closed__2; +x_15 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_13); +x_16 = l_Lean_getConstInfoCtor___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___spec__1___closed__2; +x_17 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_17, 0, x_15); +lean_ctor_set(x_17, 1, x_16); +x_18 = l_Lean_throwError___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3(x_17, x_2, x_3, x_8); +return x_18; +} +else +{ +lean_object* x_19; +lean_dec(x_2); +lean_dec(x_1); +x_19 = lean_ctor_get(x_10, 0); +lean_inc(x_19); +lean_dec(x_10); +lean_ctor_set(x_5, 0, x_19); +return x_5; +} +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_20 = lean_ctor_get(x_5, 0); +x_21 = lean_ctor_get(x_5, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_5); +x_22 = lean_ctor_get(x_20, 0); +lean_inc(x_22); +lean_dec(x_20); +lean_inc(x_1); +x_23 = lean_environment_find(x_22, x_1); +if (lean_obj_tag(x_23) == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_24 = lean_box(0); +x_25 = l_Lean_Expr_const___override(x_1, x_24); +x_26 = l_Lean_MessageData_ofExpr(x_25); +x_27 = l_Lean_getConstInfo___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__2___closed__2; +x_28 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_26); +x_29 = l_Lean_getConstInfoCtor___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___spec__1___closed__2; +x_30 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +x_31 = l_Lean_throwError___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3(x_30, x_2, x_3, x_21); +return x_31; +} +else +{ +lean_object* x_32; lean_object* x_33; +lean_dec(x_2); +lean_dec(x_1); +x_32 = lean_ctor_get(x_23, 0); +lean_inc(x_32); +lean_dec(x_23); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_21); +return x_33; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; @@ -14791,7 +14994,7 @@ LEAN_EXPORT lean_object* l_Lean_getConstInfoInduct___at___private_Lean_Server_Rp lean_object* x_5; lean_inc(x_2); lean_inc(x_1); -x_5 = l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9(x_1, x_2, x_3, x_4); +x_5 = l_Lean_getConstInfo___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__2(x_1, x_2, x_3, x_4); if (lean_obj_tag(x_5) == 0) { lean_object* x_6; @@ -14847,7 +15050,7 @@ x_19 = l_Lean_getConstInfoInduct___at___private_Lean_Server_Rpc_Deriving_0__Lean x_20 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_20, 0, x_18); lean_ctor_set(x_20, 1, x_19); -x_21 = l_Lean_throwError___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__2(x_20, x_2, x_3, x_13); +x_21 = l_Lean_throwError___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__4(x_20, x_2, x_3, x_13); return x_21; } } @@ -14877,7 +15080,7 @@ return x_25; } } } -static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__1() { +static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__1() { _start: { lean_object* x_1; @@ -14885,19 +15088,19 @@ x_1 = lean_mk_string_unchecked("instBinder", 10, 10); return x_1; } } -static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__2() { +static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___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_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__1___closed__4; x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__1___closed__10; x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__1___closed__11; -x_4 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__1; +x_4 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__1; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__3() { +static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__3() { _start: { lean_object* x_1; @@ -14905,7 +15108,7 @@ x_1 = lean_mk_string_unchecked("[", 1, 1); return x_1; } } -static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__4() { +static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -14917,11 +15120,11 @@ lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__5() { +static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__4; +x_1 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__4; x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__58; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -14929,7 +15132,7 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__6() { +static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__6() { _start: { lean_object* x_1; @@ -14937,7 +15140,7 @@ x_1 = lean_mk_string_unchecked("]", 1, 1); return x_1; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3(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_RpcEncodable_deriveInstance___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; @@ -14987,7 +15190,7 @@ x_27 = lean_ctor_get(x_25, 0); lean_inc(x_27); lean_dec(x_25); x_28 = lean_environment_main_module(x_27); -x_29 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__3; +x_29 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__3; lean_inc(x_21); lean_ctor_set_tag(x_23, 2); lean_ctor_set(x_23, 1, x_29); @@ -15002,7 +15205,7 @@ lean_ctor_set(x_32, 2, x_31); x_33 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__54; x_34 = l_Lean_addMacroScope(x_28, x_33, x_22); x_35 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__53; -x_36 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__5; +x_36 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__5; lean_inc(x_21); x_37 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_37, 0, x_21); @@ -15017,12 +15220,12 @@ x_40 = l_Lean_Syntax_node1(x_21, x_30, x_39); x_41 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__1___closed__24; lean_inc(x_21); x_42 = l_Lean_Syntax_node2(x_21, x_41, x_37, x_40); -x_43 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__6; +x_43 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__6; lean_inc(x_21); x_44 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_44, 0, x_21); lean_ctor_set(x_44, 1, x_43); -x_45 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__2; +x_45 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__2; x_46 = l_Lean_Syntax_node4(x_21, x_45, x_23, x_32, x_42, x_44); x_47 = 1; x_48 = lean_usize_add(x_2, x_47); @@ -15044,7 +15247,7 @@ x_53 = lean_ctor_get(x_51, 0); lean_inc(x_53); lean_dec(x_51); x_54 = lean_environment_main_module(x_53); -x_55 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__3; +x_55 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__3; lean_inc(x_21); x_56 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_56, 0, x_21); @@ -15059,7 +15262,7 @@ lean_ctor_set(x_59, 2, x_58); x_60 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__54; x_61 = l_Lean_addMacroScope(x_54, x_60, x_22); x_62 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___lambda__1___closed__53; -x_63 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__5; +x_63 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__5; lean_inc(x_21); x_64 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_64, 0, x_21); @@ -15074,12 +15277,12 @@ x_67 = l_Lean_Syntax_node1(x_21, x_57, x_66); x_68 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance___spec__1___closed__24; lean_inc(x_21); x_69 = l_Lean_Syntax_node2(x_21, x_68, x_64, x_67); -x_70 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__6; +x_70 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__6; lean_inc(x_21); x_71 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_71, 0, x_21); lean_ctor_set(x_71, 1, x_70); -x_72 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__2; +x_72 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__2; x_73 = l_Lean_Syntax_node4(x_21, x_72, x_56, x_59, x_69, x_71); x_74 = 1; x_75 = lean_usize_add(x_2, x_74); @@ -15118,7 +15321,7 @@ return x_81; } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__4(size_t x_1, size_t x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__6(size_t x_1, size_t x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -15142,7 +15345,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_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, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__7(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; @@ -15275,7 +15478,7 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -x_44 = l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5(x_3, x_41, x_42, x_43, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_44 = l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__7(x_3, x_41, x_42, x_43, x_5, x_6, x_7, x_8, x_9, x_10, x_11); if (lean_obj_tag(x_44) == 0) { lean_object* x_45; lean_object* x_46; @@ -15328,7 +15531,7 @@ x_17 = lean_array_size(x_15); x_18 = 0; lean_inc(x_9); lean_inc(x_7); -x_19 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3(x_17, x_18, x_15, x_5, x_6, x_7, x_8, x_9, x_10, x_16); +x_19 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5(x_17, x_18, x_15, x_5, x_6, x_7, x_8, x_9, x_10, x_16); 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; uint8_t x_26; @@ -15352,7 +15555,7 @@ if (x_26 == 0) { size_t x_27; lean_object* x_28; lean_object* x_29; x_27 = lean_array_size(x_20); -x_28 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__4(x_27, x_18, x_20); +x_28 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__6(x_27, x_18, x_20); x_29 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance(x_2, x_3, x_28, x_5, x_6, x_7, x_8, x_9, x_10, x_24); lean_dec(x_28); return x_29; @@ -15361,7 +15564,7 @@ else { size_t x_30; lean_object* x_31; lean_object* x_32; x_30 = lean_array_size(x_20); -x_31 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__4(x_30, x_18, x_20); +x_31 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__6(x_30, x_18, x_20); x_32 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveStructureInstance(x_2, x_3, x_31, x_5, x_6, x_7, x_8, x_9, x_10, x_24); lean_dec(x_10); lean_dec(x_8); @@ -15550,7 +15753,7 @@ 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_RpcEncodable_deriveInstance___lambda__3___closed__2; -x_14 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_13, x_4, x_5, x_6); +x_14 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__7(x_13, x_4, x_5, x_6); lean_dec(x_5); x_15 = !lean_is_exclusive(x_14); if (x_15 == 0) @@ -15646,7 +15849,7 @@ lean_object* x_22; lean_object* x_23; uint8_t x_24; lean_dec(x_14); lean_dec(x_12); x_22 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___closed__2; -x_23 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_22, x_2, x_3, x_15); +x_23 = l_Lean_throwError___at_Lean_withSetOptionIn___spec__7(x_22, x_2, x_3, x_15); lean_dec(x_3); x_24 = !lean_is_exclusive(x_23); if (x_24 == 0) @@ -15696,11 +15899,29 @@ return x_31; } } } -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___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___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Lean_throwError___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___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_getConstInfo___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__2(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_throwError___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__2(x_1, x_2, x_3, x_4); +x_5 = l_Lean_throwError___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__4(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } @@ -15714,7 +15935,7 @@ lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_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_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_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_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { size_t x_11; size_t x_12; lean_object* x_13; @@ -15722,7 +15943,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_RpcEncodable_deriveInstance___spec__3(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_RpcEncodable_deriveInstance___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_9); lean_dec(x_7); lean_dec(x_5); @@ -15730,7 +15951,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_RpcEncodable_deriveInstance___spec__4___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_RpcEncodable_deriveInstance___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { size_t x_4; size_t x_5; lean_object* x_6; @@ -15738,11 +15959,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_RpcEncodable_deriveInstance___spec__4(x_4, x_5, x_3); +x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__6(x_4, x_5, x_3); return x_6; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_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_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___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: { size_t x_12; size_t x_13; lean_object* x_14; @@ -15750,7 +15971,7 @@ x_12 = lean_unbox_usize(x_2); lean_dec(x_2); x_13 = lean_unbox_usize(x_3); lean_dec(x_3); -x_14 = l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5(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_foldlMUnsafe_fold___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__7(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); @@ -16551,22 +16772,26 @@ l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductive lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___closed__1); l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___closed__2 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___closed__2(); lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInductiveInstance___closed__2); +l_Lean_getConstInfo___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__2___closed__1 = _init_l_Lean_getConstInfo___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__2___closed__1(); +lean_mark_persistent(l_Lean_getConstInfo___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__2___closed__1); +l_Lean_getConstInfo___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__2___closed__2 = _init_l_Lean_getConstInfo___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__2___closed__2(); +lean_mark_persistent(l_Lean_getConstInfo___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__2___closed__2); l_Lean_getConstInfoInduct___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__1___closed__1 = _init_l_Lean_getConstInfoInduct___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__1___closed__1(); lean_mark_persistent(l_Lean_getConstInfoInduct___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__1___closed__1); l_Lean_getConstInfoInduct___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__1___closed__2 = _init_l_Lean_getConstInfoInduct___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__1___closed__2(); lean_mark_persistent(l_Lean_getConstInfoInduct___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__1___closed__2); -l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__1 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__1(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__1); -l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__2 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__2(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__2); -l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__3 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__3(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__3); -l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__4 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__4(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__4); -l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__5 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__5(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__5); -l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__6 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__6(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__3___closed__6); +l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__1 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__1(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__1); +l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__2 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__2(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__2); +l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__3 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__3(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__3); +l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__4 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__4(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__4); +l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__5 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__5(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__5); +l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__6 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__6(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___spec__5___closed__6); l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___lambda__3___closed__1 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___lambda__3___closed__1(); lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___lambda__3___closed__1); l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___lambda__3___closed__2 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncodable_deriveInstance___lambda__3___closed__2(); diff --git a/stage0/stdlib/Lean/Server/Watchdog.c b/stage0/stdlib/Lean/Server/Watchdog.c index 9cc1b58faf67..6792c7c72dfe 100644 --- a/stage0/stdlib/Lean/Server/Watchdog.c +++ b/stage0/stdlib/Lean/Server/Watchdog.c @@ -200,6 +200,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Server_Watchdog_0__Lean_Server_Watchdo lean_object* l_Lean_Json_opt___at_Lean_JsonRpc_instToJsonMessage___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_Watchdog_findDefinitions___spec__1(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_RBNode_balRight___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_groupByKey___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_IO_FS_Stream_writeLspResponse___at_Lean_Server_Watchdog_mainLoop___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_Watchdog_handleRename___spec__5(lean_object*); @@ -515,7 +516,6 @@ static lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_Watchdog_handleDid LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at_Lean_Server_Watchdog_mainLoop___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Server_References_allRefs(lean_object*); static lean_object* l_IO_FS_Stream_readNotificationAs___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__2___closed__4; -lean_object* l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleRequest___spec__7___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_Watchdog_mkLeanServerCapabilities___closed__15; LEAN_EXPORT lean_object* l_Lean_RBNode_erase___at_Lean_Server_Watchdog_ImportData_update___spec__5___boxed(lean_object*, lean_object*); @@ -17257,7 +17257,7 @@ x_18 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_18, 0, x_10); lean_ctor_set(x_18, 1, x_17); x_19 = l_Lean_Server_Watchdog_FileWorker_queuedMsgs___closed__1; -x_20 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_18, x_19); +x_20 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_18, x_19); x_21 = l_Lean_Json_mkObj(x_20); return x_21; } diff --git a/stage0/stdlib/Lean/Structure.c b/stage0/stdlib/Lean/Structure.c index cb3a1e8315a0..ddb144cd0788 100644 --- a/stage0/stdlib/Lean/Structure.c +++ b/stage0/stdlib/Lean/Structure.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Lean.Structure -// Imports: Lean.Environment Lean.ProjFns +// Imports: Lean.Environment Lean.ProjFns Lean.Exception #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -14,14 +14,19 @@ extern "C" { #endif LEAN_EXPORT lean_object* l_Lean_instInhabitedStructureInfo; +LEAN_EXPORT lean_object* l_Lean_setStructureParents___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_setStructureParents___rarg___lambda__2___closed__4; +static lean_object* l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__4; LEAN_EXPORT uint8_t l_Lean_StructureFieldInfo_lt(lean_object*, lean_object*); +static lean_object* l_Array_qsort_sort___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__5___closed__1; lean_object* l_Lean_Name_reprPrec(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getProjFnForField_x3f(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__3; static lean_object* l_Lean_getStructureCtor___closed__2; static lean_object* l_Lean_registerStructure___closed__1; -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getAllParentStructures___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__2; +static lean_object* l_Lean_registerStructure___closed__2; +LEAN_EXPORT lean_object* l_Array_binSearchAux___at_Lean_getStructureInfo_x3f___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_getStructureCtor___closed__5; LEAN_EXPORT lean_object* l_Option_repr___at___private_Lean_Structure_0__Lean_reprStructureFieldInfo____x40_Lean_Structure___hyg_64____spec__1(lean_object*, lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); @@ -31,8 +36,10 @@ LEAN_EXPORT lean_object* l_Lean_getAllParentStructures_visit(lean_object*, lean_ LEAN_EXPORT lean_object* l_Option_repr___at___private_Lean_Structure_0__Lean_reprStructureFieldInfo____x40_Lean_Structure___hyg_64____spec__2(lean_object*, lean_object*); static lean_object* l___private_Lean_Structure_0__Lean_reprStructureFieldInfo____x40_Lean_Structure___hyg_64____closed__12; LEAN_EXPORT lean_object* l_Array_binSearchAux___at_Lean_StructureInfo_getProjFn_x3f___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Structure___hyg_407____lambda__2(lean_object*); uint8_t lean_usize_dec_le(size_t, size_t); -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Structure___hyg_351____lambda__3(lean_object*); +static size_t l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__2___closed__2; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_setStructureParents___spec__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_findField_x3f___lambda__1___boxed(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_getAllParentStructures_visit___spec__1(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*); size_t lean_uint64_to_usize(uint64_t); @@ -41,19 +48,21 @@ static lean_object* l___private_Lean_Structure_0__Lean_reprStructureFieldInfo___ static lean_object* l_Option_repr___at___private_Lean_Structure_0__Lean_reprStructureFieldInfo____x40_Lean_Structure___hyg_64____spec__1___closed__3; lean_object* lean_array_push(lean_object*, lean_object*); static lean_object* l_Lean_instReprStructureFieldInfo___closed__1; +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Structure___hyg_407____lambda__2___boxed(lean_object*); lean_object* l_Array_qpartition___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__5(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_findField_x3f(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT uint8_t l_Array_contains___at_Lean_findField_x3f___spec__1(lean_object*, lean_object*); size_t lean_usize_mul(size_t, size_t); LEAN_EXPORT lean_object* l___private_Lean_Structure_0__Lean_getStructureFieldsFlattenedAux(lean_object*, lean_object*, lean_object*, uint8_t); +static lean_object* l_Lean_setStructureParents___rarg___lambda__2___closed__2; uint8_t lean_usize_dec_eq(size_t, size_t); -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_findField_x3f___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_getStructureFields___boxed(lean_object*, lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__4(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__1; lean_object* lean_environment_find(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_getStructureInfo_x3f___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_setStructureParents___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_getProjFnInfoForField_x3f___closed__1; static lean_object* l_Lean_getStructureFields___closed__2; static lean_object* l___private_Lean_Structure_0__Lean_reprStructureFieldInfo____x40_Lean_Structure___hyg_64____closed__15; @@ -61,8 +70,9 @@ static lean_object* l___private_Lean_Structure_0__Lean_reprStructureFieldInfo___ static lean_object* l___private_Lean_Structure_0__Lean_reprStructureFieldInfo____x40_Lean_Structure___hyg_64____closed__13; LEAN_EXPORT lean_object* l_Lean_getProjFnInfoForField_x3f(lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Name_quickLt(lean_object*, lean_object*); +lean_object* l_Lean_stringToMessageData(lean_object*); static lean_object* l_Array_qsort_sort___at_Lean_registerStructure___spec__2___closed__1; -LEAN_EXPORT lean_object* l_Array_binSearchAux___at_Lean_getStructureInfo_x3f___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__2___closed__3; LEAN_EXPORT lean_object* l_Lean_getProjFnForField_x3f___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_instReprStructureFieldInfo; LEAN_EXPORT lean_object* l_Lean_getPathToBaseStructureAux___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -70,6 +80,7 @@ LEAN_EXPORT lean_object* l_panic___at_Lean_getStructureFields___spec__1(lean_obj static lean_object* l_Lean_instInhabitedStructureInfo___closed__1; static lean_object* l_Lean_findField_x3f___closed__1; LEAN_EXPORT lean_object* l_Lean_mkDefaultFnOfProjFn(lean_object*); +static lean_object* l_Lean_setStructureParents___rarg___lambda__2___closed__3; LEAN_EXPORT lean_object* l_Lean_getStructureFields(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_findField_x3f___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getDefaultFnForField_x3f(lean_object*, lean_object*, lean_object*); @@ -81,51 +92,48 @@ LEAN_EXPORT lean_object* l_Lean_getFieldInfo_x3f___boxed(lean_object*, lean_obje LEAN_EXPORT lean_object* l_Lean_findField_x3f___lambda__1(lean_object*); size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Lean_isSubobjectField_x3f(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_instInhabitedStructureParentInfo; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_setStructureParents___spec__2(lean_object*, size_t, lean_object*); static lean_object* l_Lean_getStructureCtor___closed__4; static lean_object* l_Lean_instInhabitedStructureState___closed__1; static lean_object* l___private_Lean_Structure_0__Lean_reprStructureFieldInfo____x40_Lean_Structure___hyg_64____closed__23; +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__5(lean_object*, lean_object*, lean_object*); static lean_object* l_Option_repr___at___private_Lean_Structure_0__Lean_reprStructureFieldInfo____x40_Lean_Structure___hyg_64____spec__1___closed__1; -static lean_object* l_Array_qsort_sort___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__5___closed__1; -static lean_object* l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__5; static lean_object* l___private_Lean_Structure_0__Lean_reprStructureFieldInfo____x40_Lean_Structure___hyg_64____closed__16; static lean_object* l_Lean_instInhabitedStructureState___closed__2; static lean_object* l_Lean_findField_x3f___closed__2; -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_getStructureInfo_x3f___spec__2(lean_object*, size_t, lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__1; -LEAN_EXPORT lean_object* l_Array_contains___at_Lean_findField_x3f___spec__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_registerStructure___spec__1(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_StructureFieldInfo_lt___boxed(lean_object*, lean_object*); static lean_object* l_Lean_getStructureCtor___closed__6; +LEAN_EXPORT lean_object* l_Lean_setStructureParents___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_getPathToBaseStructureAux___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* l_Lean_PersistentEnvExtension_getModuleEntries___rarg(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_to_int(lean_object*); lean_object* lean_nat_div(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_registerStructure(lean_object*, lean_object*); lean_object* l_Lean_PersistentEnvExtension_addEntry___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__5___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getProjFnInfoForField_x3f___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Structure_0__Lean_reprStructureFieldInfo____x40_Lean_Structure___hyg_64____closed__3; -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_getStructureInfo_x3f___spec__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_getPathToBaseStructureAux___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Option_repr___at___private_Lean_Structure_0__Lean_reprStructureFieldInfo____x40_Lean_Structure___hyg_64____spec__1___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__7; static lean_object* l___private_Lean_Structure_0__Lean_reprStructureFieldInfo____x40_Lean_Structure___hyg_64____closed__18; +static size_t l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__2___closed__1; LEAN_EXPORT lean_object* l_Option_repr___at___private_Lean_Structure_0__Lean_reprStructureFieldInfo____x40_Lean_Structure___hyg_64____spec__2___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__3; static lean_object* l___private_Lean_Structure_0__Lean_reprStructureFieldInfo____x40_Lean_Structure___hyg_64____closed__7; LEAN_EXPORT lean_object* l_Lean_isStructureLike___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__6; static lean_object* l___private_Lean_Structure_0__Lean_reprStructureFieldInfo____x40_Lean_Structure___hyg_64____closed__9; lean_object* l_Lean_Name_append(lean_object*, lean_object*); static lean_object* l___private_Lean_Structure_0__Lean_reprStructureFieldInfo____x40_Lean_Structure___hyg_64____closed__24; LEAN_EXPORT lean_object* l_Lean_getStructureInfo_x3f(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__5___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Structure_0__Lean_reprStructureFieldInfo____x40_Lean_Structure___hyg_64____closed__22; static lean_object* l___private_Lean_Structure_0__Lean_reprStructureFieldInfo____x40_Lean_Structure___hyg_64____closed__10; -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__4(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Structure_0__Lean_reprStructureFieldInfo____x40_Lean_Structure___hyg_64____closed__2; LEAN_EXPORT lean_object* l_Lean_instInhabitedStructureDescr; LEAN_EXPORT lean_object* l_Lean_getParentStructures(lean_object*, lean_object*); -static size_t l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__2___closed__1; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insert___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Structure_0__Lean_getStructureFieldsFlattenedAux___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_name_eq(lean_object*, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); @@ -135,50 +143,49 @@ LEAN_EXPORT lean_object* l_Lean_StructureInfo_lt___boxed(lean_object*, lean_obje LEAN_EXPORT lean_object* l_Lean_isSubobjectField_x3f___boxed(lean_object*, lean_object*, lean_object*); lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_registerSimplePersistentEnvExtension___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_getStructureInfo_x3f___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__2___closed__3; -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_findField_x3f___spec__2(lean_object*, lean_object*, size_t, size_t); -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Structure___hyg_351____lambda__2___boxed(lean_object*); -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insert___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__3(size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_binSearchAux___at_Lean_getStructureInfo_x3f___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_setStructureParents(lean_object*); LEAN_EXPORT lean_object* l_Lean_StructureInfo_getProjFn_x3f___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_binSearchAux___at_Lean_StructureInfo_getProjFn_x3f___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Structure_0__Lean_reprStructureFieldInfo____x40_Lean_Structure___hyg_64____closed__25; LEAN_EXPORT lean_object* l___private_Lean_Structure_0__Lean_getStructureFieldsFlattenedAux___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__3(size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_instInhabitedStructureState; lean_object* lean_usize_to_nat(size_t); extern lean_object* l_Lean_instInhabitedProjectionFunctionInfo; uint8_t l_Lean_Environment_contains(lean_object*, lean_object*); static lean_object* l___private_Lean_Structure_0__Lean_reprStructureFieldInfo____x40_Lean_Structure___hyg_64____closed__17; -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_getStructureInfo_x3f___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getStructureInfo_x3f___boxed(lean_object*, lean_object*); extern lean_object* l_Lean_instInhabitedConstructorVal; -static lean_object* l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__4; static lean_object* l___private_Lean_Structure_0__Lean_reprStructureFieldInfo____x40_Lean_Structure___hyg_64____closed__20; static lean_object* l_Lean_getStructureFields___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Structure_0__Lean_reprStructureFieldInfo____x40_Lean_Structure___hyg_64_(lean_object*, lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__6; static lean_object* l_Lean_instInhabitedStructureDescr___closed__1; LEAN_EXPORT lean_object* l_Lean_getFieldInfo_x3f(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Structure_0__Lean_getStructureFieldsFlattenedAux___spec__1(lean_object*, lean_object*, uint8_t, lean_object*, size_t, size_t, lean_object*); -static size_t l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__2___closed__2; +lean_object* l_Lean_throwError___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getPathToBaseStructureAux(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Structure_0__Lean_reprStructureFieldInfo____x40_Lean_Structure___hyg_64____closed__11; lean_object* lean_string_length(lean_object*); static lean_object* l_Lean_findField_x3f___closed__3; -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_getStructureInfo_x3f___spec__1___boxed(lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_binSearchAux___at_Lean_getStructureInfo_x3f___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_3025_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_getParentStructures___spec__1(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Structure___hyg_351_(lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__5; static lean_object* l_Lean_mkDefaultFnOfProjFn___closed__2; lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_instInhabitedStructureFieldInfo; lean_object* l___private_Lean_Expr_0__Lean_reprBinderInfo____x40_Lean_Expr___hyg_422_(uint8_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Structure___hyg_407_(lean_object*); +static lean_object* l_Lean_instInhabitedStructureParentInfo___closed__1; lean_object* l_Lean_PersistentHashMap_mkEmptyEntries(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_findField_x3f___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint64_t l_Lean_Name_hash___override(lean_object*); +uint8_t l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(lean_object*, lean_object*); lean_object* l_Repr_addAppParen(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getAllParentStructures(lean_object*, lean_object*); lean_object* lean_panic_fn(lean_object*, lean_object*); static lean_object* l_Lean_getStructureCtor___closed__1; @@ -186,21 +193,21 @@ LEAN_EXPORT lean_object* l___private_Lean_Structure_0__Lean_reprStructureFieldIn lean_object* lean_nat_sub(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_isStructure(lean_object*, lean_object*); static lean_object* l___private_Lean_Structure_0__Lean_reprStructureFieldInfo____x40_Lean_Structure___hyg_64____closed__8; +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Structure___hyg_407____lambda__1(lean_object*, lean_object*); lean_object* l_Lean_SimplePersistentEnvExtension_getState___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_getStructureCtor___closed__3; lean_object* l_Lean_PersistentHashMap_mkCollisionNode___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_findField_x3f___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_isStructure___boxed(lean_object*, lean_object*); lean_object* l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); lean_object* l_Lean_Environment_getModuleIdxFor_x3f(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Structure___hyg_351____lambda__1(lean_object*, lean_object*); static lean_object* l_Option_repr___at___private_Lean_Structure_0__Lean_reprStructureFieldInfo____x40_Lean_Structure___hyg_64____spec__1___closed__2; lean_object* l_List_reverse___rarg(lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__7; static lean_object* l_Lean_instInhabitedStructureInfo___closed__2; -static lean_object* l_Lean_getStructureInfo_x3f___closed__2; size_t lean_usize_sub(size_t, size_t); static lean_object* l___private_Lean_Structure_0__Lean_reprStructureFieldInfo____x40_Lean_Structure___hyg_64____closed__6; lean_object* lean_array_mk(lean_object*); +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Structure___hyg_407____lambda__3(lean_object*); LEAN_EXPORT lean_object* l_Lean_getStructureCtor(lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_getAllParentStructures_visit___boxed(lean_object*, lean_object*, lean_object*); @@ -213,30 +220,34 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_getAllParentStructur size_t lean_usize_shift_left(size_t, size_t); static lean_object* l___private_Lean_Structure_0__Lean_reprStructureFieldInfo____x40_Lean_Structure___hyg_64____closed__4; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_registerStructure___spec__1___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_setStructureParents___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*); static lean_object* l_Lean_getStructureInfo_x3f___closed__1; static lean_object* l___private_Lean_Structure_0__Lean_reprStructureFieldInfo____x40_Lean_Structure___hyg_64____closed__1; LEAN_EXPORT lean_object* l_Lean_structureExt; lean_object* lean_array_get_size(lean_object*); static lean_object* l_Lean_instInhabitedStructureFieldInfo___closed__1; +static lean_object* l_Lean_setStructureParents___rarg___lambda__2___closed__1; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_setStructureParents___spec__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_registerStructure___spec__2(lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_StructureInfo_getProjFn_x3f(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_setStructureParents___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); lean_object* l_Lean_PersistentHashMap_getCollisionNodeSize___rarg(lean_object*); LEAN_EXPORT uint8_t l_Lean_StructureInfo_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getStructureFieldsFlattened(lean_object*, lean_object*, uint8_t); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_findField_x3f___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* lean_array_uset(lean_object*, size_t, lean_object*); +lean_object* l_Lean_MessageData_ofName(lean_object*); lean_object* lean_array_get(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_setStructureParents___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getParentStructures___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getStructureFieldsFlattened___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_isStructureLike(lean_object*, lean_object*); static lean_object* l___private_Lean_Structure_0__Lean_reprStructureFieldInfo____x40_Lean_Structure___hyg_64____closed__19; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_findField_x3f___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_setStructureParents___rarg___lambda__1(lean_object*, lean_object*, lean_object*); size_t lean_usize_land(size_t, size_t); -static lean_object* l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__2; -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Structure___hyg_351____lambda__2(lean_object*); static lean_object* _init_l_Lean_instInhabitedStructureFieldInfo___closed__1() { _start: { @@ -787,6 +798,27 @@ x_4 = lean_box(x_3); return x_4; } } +static lean_object* _init_l_Lean_instInhabitedStructureParentInfo___closed__1() { +_start: +{ +lean_object* x_1; uint8_t x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = 0; +x_3 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_1); +lean_ctor_set_uint8(x_3, sizeof(void*)*2, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_instInhabitedStructureParentInfo() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_instInhabitedStructureParentInfo___closed__1; +return x_1; +} +} static lean_object* _init_l_Lean_instInhabitedStructureInfo___closed__1() { _start: { @@ -802,10 +834,11 @@ static lean_object* _init_l_Lean_instInhabitedStructureInfo___closed__2() { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); x_2 = l_Lean_instInhabitedStructureInfo___closed__1; -x_3 = lean_alloc_ctor(0, 3, 0); +x_3 = lean_alloc_ctor(0, 4, 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); return x_3; } } @@ -1047,7 +1080,7 @@ x_1 = l_Lean_instInhabitedStructureState___closed__2; return x_1; } } -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_initFn____x40_Lean_Structure___hyg_351____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) { +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__3(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; uint8_t x_8; @@ -1074,7 +1107,7 @@ x_17 = lean_usize_shift_right(x_12, x_16); x_18 = lean_unsigned_to_nat(1u); x_19 = lean_nat_add(x_5, x_18); lean_dec(x_5); -x_20 = l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__2(x_6, x_17, x_1, x_9, x_10); +x_20 = l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__2(x_6, x_17, x_1, x_9, x_10); x_4 = lean_box(0); x_5 = x_19; x_6 = x_20; @@ -1082,7 +1115,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; @@ -1174,7 +1207,7 @@ return x_29; } } } -static size_t _init_l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__2___closed__1() { +static size_t _init_l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__2___closed__1() { _start: { size_t x_1; size_t x_2; size_t x_3; @@ -1184,17 +1217,17 @@ x_3 = lean_usize_shift_left(x_1, x_2); return x_3; } } -static size_t _init_l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__2___closed__2() { +static size_t _init_l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__2___closed__2() { _start: { size_t x_1; size_t x_2; size_t x_3; x_1 = 1; -x_2 = l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__2___closed__1; +x_2 = l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__2___closed__1; x_3 = lean_usize_sub(x_2, x_1); return x_3; } } -static lean_object* _init_l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__2___closed__3() { +static lean_object* _init_l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__2___closed__3() { _start: { lean_object* x_1; @@ -1202,7 +1235,7 @@ x_1 = l_Lean_PersistentHashMap_mkEmptyEntries(lean_box(0), lean_box(0)); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__2(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__2(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5) { _start: { if (lean_obj_tag(x_1) == 0) @@ -1215,7 +1248,7 @@ lean_object* x_7; size_t x_8; size_t x_9; size_t x_10; size_t x_11; lean_object* x_7 = lean_ctor_get(x_1, 0); x_8 = 1; x_9 = 5; -x_10 = l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__2___closed__2; +x_10 = l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__2___closed__2; x_11 = lean_usize_land(x_2, x_10); x_12 = lean_usize_to_nat(x_11); x_13 = lean_array_get_size(x_7); @@ -1315,7 +1348,7 @@ lean_object* x_35; size_t x_36; size_t x_37; lean_object* x_38; lean_object* x_3 x_35 = lean_ctor_get(x_15, 0); x_36 = lean_usize_shift_right(x_2, x_9); x_37 = lean_usize_add(x_3, x_8); -x_38 = l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__2(x_35, x_36, x_37, x_4, x_5); +x_38 = l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__2(x_35, x_36, x_37, x_4, x_5); lean_ctor_set(x_15, 0, x_38); x_39 = lean_array_fset(x_17, x_12, x_15); lean_dec(x_12); @@ -1330,7 +1363,7 @@ lean_inc(x_40); lean_dec(x_15); x_41 = lean_usize_shift_right(x_2, x_9); x_42 = lean_usize_add(x_3, x_8); -x_43 = l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__2(x_40, x_41, x_42, x_4, x_5); +x_43 = l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__2(x_40, x_41, x_42, x_4, x_5); x_44 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_44, 0, x_43); x_45 = lean_array_fset(x_17, x_12, x_44); @@ -1361,7 +1394,7 @@ lean_inc(x_48); lean_dec(x_1); x_49 = 1; x_50 = 5; -x_51 = l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__2___closed__2; +x_51 = l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__2___closed__2; x_52 = lean_usize_land(x_2, x_51); x_53 = lean_usize_to_nat(x_52); x_54 = lean_array_get_size(x_48); @@ -1446,7 +1479,7 @@ if (lean_is_exclusive(x_57)) { } x_73 = lean_usize_shift_right(x_2, x_50); x_74 = lean_usize_add(x_3, x_49); -x_75 = l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__2(x_71, x_73, x_74, x_4, x_5); +x_75 = l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__2(x_71, x_73, x_74, x_4, x_5); if (lean_is_scalar(x_72)) { x_76 = lean_alloc_ctor(1, 1, 0); } else { @@ -1483,7 +1516,7 @@ if (x_82 == 0) { lean_object* x_83; lean_object* x_84; size_t x_85; uint8_t x_86; x_83 = lean_unsigned_to_nat(0u); -x_84 = l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__4(x_1, x_83, x_4, x_5); +x_84 = l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__4(x_1, x_83, x_4, x_5); x_85 = 7; x_86 = lean_usize_dec_le(x_85, x_3); if (x_86 == 0) @@ -1501,8 +1534,8 @@ lean_inc(x_90); x_91 = lean_ctor_get(x_84, 1); lean_inc(x_91); lean_dec(x_84); -x_92 = l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__2___closed__3; -x_93 = l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__3(x_3, x_90, x_91, lean_box(0), x_83, x_92); +x_92 = l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__2___closed__3; +x_93 = l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__3(x_3, x_90, x_91, lean_box(0), x_83, x_92); lean_dec(x_91); lean_dec(x_90); return x_93; @@ -1529,7 +1562,7 @@ x_96 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_96, 0, x_94); lean_ctor_set(x_96, 1, x_95); x_97 = lean_unsigned_to_nat(0u); -x_98 = l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__4(x_96, x_97, x_4, x_5); +x_98 = l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__4(x_96, x_97, x_4, x_5); x_99 = 7; x_100 = lean_usize_dec_le(x_99, x_3); if (x_100 == 0) @@ -1547,8 +1580,8 @@ lean_inc(x_104); x_105 = lean_ctor_get(x_98, 1); lean_inc(x_105); lean_dec(x_98); -x_106 = l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__2___closed__3; -x_107 = l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__3(x_3, x_104, x_105, lean_box(0), x_97, x_106); +x_106 = l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__2___closed__3; +x_107 = l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__3(x_3, x_104, x_105, lean_box(0), x_97, x_106); lean_dec(x_105); lean_dec(x_104); return x_107; @@ -1566,18 +1599,18 @@ return x_98; } } } -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insert___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insert___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint64_t x_4; size_t x_5; size_t x_6; lean_object* x_7; x_4 = l_Lean_Name_hash___override(x_2); x_5 = lean_uint64_to_usize(x_4); x_6 = 1; -x_7 = l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__2(x_1, x_5, x_6, x_2, x_3); +x_7 = l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__2(x_1, x_5, x_6, x_2, x_3); return x_7; } } -static lean_object* _init_l_Array_qsort_sort___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__5___closed__1() { +static lean_object* _init_l_Array_qsort_sort___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__5___closed__1() { _start: { lean_object* x_1; @@ -1585,7 +1618,7 @@ x_1 = lean_alloc_closure((void*)(l_Lean_StructureInfo_lt___boxed), 2, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -1598,7 +1631,7 @@ return x_1; else { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; -x_5 = l_Array_qsort_sort___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__5___closed__1; +x_5 = l_Array_qsort_sort___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__5___closed__1; lean_inc(x_2); x_6 = l_Array_qpartition___rarg(x_1, x_5, x_2, x_3); x_7 = lean_ctor_get(x_6, 0); @@ -1610,7 +1643,7 @@ x_9 = lean_nat_dec_le(x_3, x_7); if (x_9 == 0) { lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_10 = l_Array_qsort_sort___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__5(x_8, x_2, x_7); +x_10 = l_Array_qsort_sort___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__5(x_8, x_2, x_7); x_11 = lean_unsigned_to_nat(1u); x_12 = lean_nat_add(x_7, x_11); lean_dec(x_7); @@ -1627,17 +1660,17 @@ return x_8; } } } -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Structure___hyg_351____lambda__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Structure___hyg_407____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); -x_4 = l_Lean_PersistentHashMap_insert___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__1(x_1, x_3, x_2); +x_4 = l_Lean_PersistentHashMap_insert___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__1(x_1, x_3, x_2); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Structure___hyg_351____lambda__2(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Structure___hyg_407____lambda__2(lean_object* x_1) { _start: { lean_object* x_2; @@ -1645,7 +1678,7 @@ x_2 = l_Lean_instInhabitedStructureState___closed__2; return x_2; } } -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Structure___hyg_351____lambda__3(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Structure___hyg_407____lambda__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; @@ -1655,12 +1688,12 @@ x_4 = lean_unsigned_to_nat(1u); x_5 = lean_nat_sub(x_3, x_4); lean_dec(x_3); x_6 = lean_unsigned_to_nat(0u); -x_7 = l_Array_qsort_sort___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__5(x_2, x_6, x_5); +x_7 = l_Array_qsort_sort___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__5(x_2, x_6, x_5); lean_dec(x_5); return x_7; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__1() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__1() { _start: { lean_object* x_1; @@ -1668,7 +1701,7 @@ x_1 = lean_mk_string_unchecked("Lean", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__2() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__2() { _start: { lean_object* x_1; @@ -1676,48 +1709,48 @@ x_1 = lean_mk_string_unchecked("structureExt", 12, 12); return x_1; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__3() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__1; -x_2 = l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__2; +x_1 = l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__1; +x_2 = l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__2; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__4() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__4() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_initFn____x40_Lean_Structure___hyg_351____lambda__1), 2, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_initFn____x40_Lean_Structure___hyg_407____lambda__1), 2, 0); return x_1; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__5() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__5() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_initFn____x40_Lean_Structure___hyg_351____lambda__2___boxed), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_initFn____x40_Lean_Structure___hyg_407____lambda__2___boxed), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__6() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__6() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_initFn____x40_Lean_Structure___hyg_351____lambda__3), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_initFn____x40_Lean_Structure___hyg_407____lambda__3), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__7() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Structure___hyg_407____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_initFn____x40_Lean_Structure___hyg_351____closed__3; -x_2 = l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__4; -x_3 = l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__5; -x_4 = l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__6; +x_1 = l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__3; +x_2 = l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__4; +x_3 = l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__5; +x_4 = l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__6; x_5 = lean_alloc_ctor(0, 4, 0); lean_ctor_set(x_5, 0, x_1); lean_ctor_set(x_5, 1, x_2); @@ -1726,28 +1759,28 @@ lean_ctor_set(x_5, 3, x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Structure___hyg_351_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Structure___hyg_407_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__7; +x_2 = l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__7; x_3 = l_Lean_registerSimplePersistentEnvExtension___rarg(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_initFn____x40_Lean_Structure___hyg_351____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_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { size_t x_7; lean_object* x_8; x_7 = lean_unbox_usize(x_1); lean_dec(x_1); -x_8 = l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__3(x_7, x_2, x_3, x_4, x_5, x_6); +x_8 = l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__3(x_7, x_2, x_3, x_4, x_5, x_6); lean_dec(x_3); lean_dec(x_2); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { size_t x_6; size_t x_7; lean_object* x_8; @@ -1755,24 +1788,24 @@ x_6 = lean_unbox_usize(x_2); lean_dec(x_2); x_7 = lean_unbox_usize(x_3); lean_dec(x_3); -x_8 = l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__2(x_1, x_6, x_7, x_4, x_5); +x_8 = l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__2(x_1, x_6, x_7, x_4, x_5); return x_8; } } -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Array_qsort_sort___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__5(x_1, x_2, x_3); +x_4 = l_Array_qsort_sort___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__5(x_1, x_2, x_3); lean_dec(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Structure___hyg_351____lambda__2___boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Structure___hyg_407____lambda__2___boxed(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l_Lean_initFn____x40_Lean_Structure___hyg_351____lambda__2(x_1); +x_2 = l_Lean_initFn____x40_Lean_Structure___hyg_407____lambda__2(x_1); lean_dec(x_1); return x_2; } @@ -1877,6 +1910,15 @@ return x_8; static lean_object* _init_l_Lean_registerStructure___closed__1() { _start: { +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_array_mk(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_registerStructure___closed__2() { +_start: +{ lean_object* x_1; x_1 = l_Lean_structureExt; return x_1; @@ -1885,7 +1927,7 @@ return x_1; LEAN_EXPORT lean_object* l_Lean_registerStructure(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_3; lean_object* x_4; size_t x_5; size_t x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +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; x_3 = lean_ctor_get(x_2, 0); lean_inc(x_3); x_4 = lean_ctor_get(x_2, 1); @@ -1902,13 +1944,15 @@ lean_dec(x_8); x_11 = lean_unsigned_to_nat(0u); x_12 = l_Array_qsort_sort___at_Lean_registerStructure___spec__2(x_4, x_11, x_10); lean_dec(x_10); -x_13 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_13, 0, x_3); -lean_ctor_set(x_13, 1, x_7); -lean_ctor_set(x_13, 2, x_12); -x_14 = l_Lean_registerStructure___closed__1; -x_15 = l_Lean_PersistentEnvExtension_addEntry___rarg(x_14, x_1, x_13); -return x_15; +x_13 = l_Lean_registerStructure___closed__1; +x_14 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_14, 0, x_3); +lean_ctor_set(x_14, 1, x_7); +lean_ctor_set(x_14, 2, x_12); +lean_ctor_set(x_14, 3, x_13); +x_15 = l_Lean_registerStructure___closed__2; +x_16 = l_Lean_PersistentEnvExtension_addEntry___rarg(x_15, x_1, x_14); +return x_16; } } LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_registerStructure___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { @@ -1932,7 +1976,7 @@ lean_dec(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_getStructureInfo_x3f___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_setStructureParents___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; uint8_t x_7; @@ -1974,7 +2018,7 @@ return x_15; } } } -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_getStructureInfo_x3f___spec__2(lean_object* x_1, size_t x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_setStructureParents___spec__2(lean_object* x_1, size_t x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_1) == 0) @@ -1986,7 +2030,7 @@ if (x_4 == 0) lean_object* x_5; size_t x_6; size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; x_5 = lean_ctor_get(x_1, 0); x_6 = 5; -x_7 = l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__2___closed__2; +x_7 = l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__2___closed__2; x_8 = lean_usize_land(x_2, x_7); x_9 = lean_usize_to_nat(x_8); x_10 = lean_box(2); @@ -2047,7 +2091,7 @@ x_20 = lean_ctor_get(x_1, 0); lean_inc(x_20); lean_dec(x_1); x_21 = 5; -x_22 = l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__2___closed__2; +x_22 = l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__2___closed__2; x_23 = lean_usize_land(x_2, x_22); x_24 = lean_usize_to_nat(x_23); x_25 = lean_box(2); @@ -2109,24 +2153,205 @@ x_37 = lean_ctor_get(x_1, 1); lean_inc(x_37); lean_dec(x_1); x_38 = lean_unsigned_to_nat(0u); -x_39 = l_Lean_PersistentHashMap_findAtAux___at_Lean_getStructureInfo_x3f___spec__3(x_36, x_37, lean_box(0), x_38, x_3); +x_39 = l_Lean_PersistentHashMap_findAtAux___at_Lean_setStructureParents___spec__3(x_36, x_37, lean_box(0), x_38, x_3); lean_dec(x_37); lean_dec(x_36); return x_39; } } } -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_getStructureInfo_x3f___spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_setStructureParents___spec__1(lean_object* x_1, lean_object* x_2) { _start: { uint64_t x_3; size_t x_4; lean_object* x_5; x_3 = l_Lean_Name_hash___override(x_2); x_4 = lean_uint64_to_usize(x_3); -x_5 = l_Lean_PersistentHashMap_findAux___at_Lean_getStructureInfo_x3f___spec__2(x_1, x_4, x_2); +x_5 = l_Lean_PersistentHashMap_findAux___at_Lean_setStructureParents___spec__2(x_1, x_4, x_2); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_setStructureParents___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +uint8_t x_4; +x_4 = !lean_is_exclusive(x_1); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_5 = lean_ctor_get(x_1, 3); +lean_dec(x_5); +lean_ctor_set(x_1, 3, x_2); +x_6 = l_Lean_registerStructure___closed__2; +x_7 = l_Lean_PersistentEnvExtension_addEntry___rarg(x_6, x_3, x_1); +return x_7; +} +else +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_8 = lean_ctor_get(x_1, 0); +x_9 = lean_ctor_get(x_1, 1); +x_10 = lean_ctor_get(x_1, 2); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_dec(x_1); +x_11 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_11, 0, x_8); +lean_ctor_set(x_11, 1, x_9); +lean_ctor_set(x_11, 2, x_10); +lean_ctor_set(x_11, 3, x_2); +x_12 = l_Lean_registerStructure___closed__2; +x_13 = l_Lean_PersistentEnvExtension_addEntry___rarg(x_12, x_3, x_11); +return x_13; +} +} +} +static lean_object* _init_l_Lean_setStructureParents___rarg___lambda__2___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("cannot set structure parents for '", 34, 34); +return x_1; +} +} +static lean_object* _init_l_Lean_setStructureParents___rarg___lambda__2___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_setStructureParents___rarg___lambda__2___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_setStructureParents___rarg___lambda__2___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("', structure not defined in current module", 42, 42); +return x_1; +} +} +static lean_object* _init_l_Lean_setStructureParents___rarg___lambda__2___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_setStructureParents___rarg___lambda__2___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_setStructureParents___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 = l_Lean_instInhabitedStructureState; +x_8 = l_Lean_registerStructure___closed__2; +x_9 = l_Lean_SimplePersistentEnvExtension_getState___rarg(x_7, x_8, x_6); +x_10 = l_Lean_PersistentHashMap_find_x3f___at_Lean_setStructureParents___spec__1(x_9, x_1); +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_dec(x_5); +lean_dec(x_4); +x_11 = l_Lean_MessageData_ofName(x_1); +x_12 = l_Lean_setStructureParents___rarg___lambda__2___closed__2; +x_13 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_11); +x_14 = l_Lean_setStructureParents___rarg___lambda__2___closed__4; +x_15 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_15, 0, x_13); +lean_ctor_set(x_15, 1, x_14); +x_16 = l_Lean_throwError___rarg(x_2, x_3, x_15); +return x_16; +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_17 = lean_ctor_get(x_10, 0); +lean_inc(x_17); +lean_dec(x_10); +x_18 = lean_ctor_get(x_4, 1); +lean_inc(x_18); +lean_dec(x_4); +x_19 = lean_alloc_closure((void*)(l_Lean_setStructureParents___rarg___lambda__1), 3, 2); +lean_closure_set(x_19, 0, x_17); +lean_closure_set(x_19, 1, x_5); +x_20 = lean_apply_1(x_18, x_19); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Lean_setStructureParents___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_6 = lean_ctor_get(x_1, 1); +lean_inc(x_6); +x_7 = lean_ctor_get(x_2, 0); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_Lean_setStructureParents___rarg___lambda__2___boxed), 6, 5); +lean_closure_set(x_8, 0, x_4); +lean_closure_set(x_8, 1, x_1); +lean_closure_set(x_8, 2, x_3); +lean_closure_set(x_8, 3, x_2); +lean_closure_set(x_8, 4, x_5); +x_9 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_7, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_setStructureParents(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_setStructureParents___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_setStructureParents___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; +x_6 = l_Lean_PersistentHashMap_findAtAux___at_Lean_setStructureParents___spec__3(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_5); +lean_dec(x_2); +lean_dec(x_1); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_setStructureParents___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; lean_object* x_5; +x_4 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_5 = l_Lean_PersistentHashMap_findAux___at_Lean_setStructureParents___spec__2(x_1, x_4, x_3); +lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Array_binSearchAux___at_Lean_getStructureInfo_x3f___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_setStructureParents___spec__1___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Lean_PersistentHashMap_find_x3f___at_Lean_setStructureParents___spec__1(x_1, x_2); +lean_dec(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_setStructureParents___rarg___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; +x_7 = l_Lean_setStructureParents___rarg___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6); +lean_dec(x_6); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_binSearchAux___at_Lean_getStructureInfo_x3f___spec__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_6; @@ -2217,15 +2442,6 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_getStructureInfo_x3f___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = lean_box(0); -x_2 = lean_array_mk(x_1); -return x_2; -} -} LEAN_EXPORT lean_object* l_Lean_getStructureInfo_x3f(lean_object* x_1, lean_object* x_2) { _start: { @@ -2235,9 +2451,9 @@ if (lean_obj_tag(x_3) == 0) { lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_4 = l_Lean_instInhabitedStructureState; -x_5 = l_Lean_registerStructure___closed__1; +x_5 = l_Lean_registerStructure___closed__2; x_6 = l_Lean_SimplePersistentEnvExtension_getState___rarg(x_4, x_5, x_1); -x_7 = l_Lean_PersistentHashMap_find_x3f___at_Lean_getStructureInfo_x3f___spec__1(x_6, x_2); +x_7 = l_Lean_PersistentHashMap_find_x3f___at_Lean_setStructureParents___spec__1(x_6, x_2); lean_dec(x_2); return x_7; } @@ -2248,14 +2464,15 @@ x_8 = lean_ctor_get(x_3, 0); lean_inc(x_8); lean_dec(x_3); x_9 = l_Lean_getStructureInfo_x3f___closed__1; -x_10 = l_Lean_registerStructure___closed__1; +x_10 = l_Lean_registerStructure___closed__2; x_11 = l_Lean_PersistentEnvExtension_getModuleEntries___rarg(x_9, x_10, x_1, x_8); lean_dec(x_8); -x_12 = l_Lean_getStructureInfo_x3f___closed__2; -x_13 = lean_alloc_ctor(0, 3, 0); +x_12 = l_Lean_registerStructure___closed__1; +x_13 = lean_alloc_ctor(0, 4, 0); lean_ctor_set(x_13, 0, x_2); lean_ctor_set(x_13, 1, x_12); lean_ctor_set(x_13, 2, x_12); +lean_ctor_set(x_13, 3, x_12); x_14 = lean_array_get_size(x_11); x_15 = lean_unsigned_to_nat(1u); x_16 = lean_nat_sub(x_14, x_15); @@ -2275,49 +2492,18 @@ else { lean_object* x_20; lean_object* x_21; x_20 = lean_box(0); -x_21 = l_Array_binSearchAux___at_Lean_getStructureInfo_x3f___spec__4(x_20, x_11, x_13, x_17, x_16); +x_21 = l_Array_binSearchAux___at_Lean_getStructureInfo_x3f___spec__1(x_20, x_11, x_13, x_17, x_16); lean_dec(x_11); return x_21; } } } } -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_getStructureInfo_x3f___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_Array_binSearchAux___at_Lean_getStructureInfo_x3f___spec__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_PersistentHashMap_findAtAux___at_Lean_getStructureInfo_x3f___spec__3(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_5); -lean_dec(x_2); -lean_dec(x_1); -return x_6; -} -} -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_getStructureInfo_x3f___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -size_t x_4; lean_object* x_5; -x_4 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_5 = l_Lean_PersistentHashMap_findAux___at_Lean_getStructureInfo_x3f___spec__2(x_1, x_4, x_3); -lean_dec(x_3); -return x_5; -} -} -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_getStructureInfo_x3f___spec__1___boxed(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = l_Lean_PersistentHashMap_find_x3f___at_Lean_getStructureInfo_x3f___spec__1(x_1, x_2); -lean_dec(x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Array_binSearchAux___at_Lean_getStructureInfo_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_Array_binSearchAux___at_Lean_getStructureInfo_x3f___spec__4(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Array_binSearchAux___at_Lean_getStructureInfo_x3f___spec__1(x_1, x_2, x_3, x_4, x_5); lean_dec(x_2); lean_dec(x_1); return x_6; @@ -2371,7 +2557,7 @@ static lean_object* _init_l_Lean_getStructureCtor___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_getStructureCtor___closed__1; x_2 = l_Lean_getStructureCtor___closed__2; -x_3 = lean_unsigned_to_nat(76u); +x_3 = lean_unsigned_to_nat(131u); x_4 = lean_unsigned_to_nat(9u); x_5 = l_Lean_getStructureCtor___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -2392,7 +2578,7 @@ static lean_object* _init_l_Lean_getStructureCtor___closed__6() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_getStructureCtor___closed__1; x_2 = l_Lean_getStructureCtor___closed__2; -x_3 = lean_unsigned_to_nat(75u); +x_3 = lean_unsigned_to_nat(130u); x_4 = lean_unsigned_to_nat(11u); x_5 = l_Lean_getStructureCtor___closed__5; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -2542,7 +2728,7 @@ static lean_object* _init_l_Lean_getStructureFields___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_getStructureCtor___closed__1; x_2 = l_Lean_getStructureFields___closed__1; -x_3 = lean_unsigned_to_nat(83u); +x_3 = lean_unsigned_to_nat(138u); x_4 = lean_unsigned_to_nat(4u); x_5 = l_Lean_getStructureCtor___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -2732,7 +2918,7 @@ lean_object* x_7; lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_7 = l_Lean_getStructureInfo_x3f___closed__2; +x_7 = l_Lean_registerStructure___closed__1; return x_7; } else @@ -2745,7 +2931,7 @@ lean_object* x_9; lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_9 = l_Lean_getStructureInfo_x3f___closed__2; +x_9 = l_Lean_registerStructure___closed__1; return x_9; } else @@ -2754,7 +2940,7 @@ size_t x_10; size_t x_11; lean_object* x_12; lean_object* x_13; x_10 = 0; x_11 = lean_usize_of_nat(x_4); lean_dec(x_4); -x_12 = l_Lean_getStructureInfo_x3f___closed__2; +x_12 = l_Lean_registerStructure___closed__1; x_13 = l_Array_foldlMUnsafe_fold___at_Lean_getParentStructures___spec__1(x_1, x_2, x_3, x_10, x_11, x_12); lean_dec(x_3); return x_13; @@ -2878,7 +3064,7 @@ LEAN_EXPORT lean_object* l_Lean_getAllParentStructures(lean_object* x_1, lean_ob _start: { lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_3 = l_Lean_getStructureInfo_x3f___closed__2; +x_3 = l_Lean_registerStructure___closed__1; x_4 = l_Lean_getAllParentStructures_visit(x_1, x_2, x_3); x_5 = lean_ctor_get(x_4, 1); lean_inc(x_5); @@ -2895,66 +3081,7 @@ lean_dec(x_1); return x_3; } } -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_findField_x3f___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_6, x_1); -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_findField_x3f___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 -{ -size_t x_7; size_t x_8; uint8_t x_9; -x_7 = 0; -x_8 = lean_usize_of_nat(x_3); -lean_dec(x_3); -x_9 = l_Array_anyMUnsafe_any___at_Lean_findField_x3f___spec__2(x_2, x_1, x_7, x_8); -return x_9; -} -} -} -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_findField_x3f___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_findField_x3f___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7) { _start: { uint8_t x_8; @@ -3061,7 +3188,7 @@ LEAN_EXPORT lean_object* l_Lean_findField_x3f(lean_object* x_1, lean_object* x_2 lean_object* x_4; uint8_t x_5; lean_inc(x_2); x_4 = l_Lean_getStructureFields(x_1, x_2); -x_5 = l_Array_contains___at_Lean_findField_x3f___spec__1(x_4, x_3); +x_5 = l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(x_4, x_3); lean_dec(x_4); if (x_5 == 0) { @@ -3070,7 +3197,7 @@ x_6 = l_Lean_getParentStructures(x_1, x_2); x_7 = lean_array_size(x_6); x_8 = 0; x_9 = l_Lean_findField_x3f___closed__1; -x_10 = l_Array_forInUnsafe_loop___at_Lean_findField_x3f___spec__3(x_1, x_3, x_9, x_6, x_7, x_8, x_9); +x_10 = l_Array_forInUnsafe_loop___at_Lean_findField_x3f___spec__1(x_1, x_3, x_9, x_6, x_7, x_8, x_9); lean_dec(x_6); x_11 = lean_ctor_get(x_10, 0); lean_inc(x_11); @@ -3099,33 +3226,7 @@ return x_14; } } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_findField_x3f___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_findField_x3f___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_findField_x3f___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_findField_x3f___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_forInUnsafe_loop___at_Lean_findField_x3f___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_findField_x3f___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { size_t x_8; size_t x_9; lean_object* x_10; @@ -3133,7 +3234,7 @@ x_8 = lean_unbox_usize(x_5); lean_dec(x_5); x_9 = lean_unbox_usize(x_6); lean_dec(x_6); -x_10 = l_Array_forInUnsafe_loop___at_Lean_findField_x3f___spec__3(x_1, x_2, x_3, x_4, x_8, x_9, x_7); +x_10 = l_Array_forInUnsafe_loop___at_Lean_findField_x3f___spec__1(x_1, x_2, x_3, x_4, x_8, x_9, x_7); lean_dec(x_7); lean_dec(x_4); lean_dec(x_3); @@ -3289,7 +3390,7 @@ LEAN_EXPORT lean_object* l_Lean_getStructureFieldsFlattened(lean_object* x_1, le _start: { lean_object* x_4; lean_object* x_5; -x_4 = l_Lean_getStructureInfo_x3f___closed__2; +x_4 = l_Lean_registerStructure___closed__1; x_5 = l___private_Lean_Structure_0__Lean_getStructureFieldsFlattenedAux(x_1, x_2, x_4, x_3); return x_5; } @@ -4059,6 +4160,7 @@ return x_24; } lean_object* initialize_Lean_Environment(uint8_t builtin, lean_object*); lean_object* initialize_Lean_ProjFns(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Exception(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Lean_Structure(uint8_t builtin, lean_object* w) { lean_object * res; @@ -4070,6 +4172,9 @@ lean_dec_ref(res); res = initialize_Lean_ProjFns(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +res = initialize_Lean_Exception(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_instInhabitedStructureFieldInfo___closed__1 = _init_l_Lean_instInhabitedStructureFieldInfo___closed__1(); lean_mark_persistent(l_Lean_instInhabitedStructureFieldInfo___closed__1); l_Lean_instInhabitedStructureFieldInfo = _init_l_Lean_instInhabitedStructureFieldInfo(); @@ -4136,6 +4241,10 @@ l_Lean_instReprStructureFieldInfo___closed__1 = _init_l_Lean_instReprStructureFi lean_mark_persistent(l_Lean_instReprStructureFieldInfo___closed__1); l_Lean_instReprStructureFieldInfo = _init_l_Lean_instReprStructureFieldInfo(); lean_mark_persistent(l_Lean_instReprStructureFieldInfo); +l_Lean_instInhabitedStructureParentInfo___closed__1 = _init_l_Lean_instInhabitedStructureParentInfo___closed__1(); +lean_mark_persistent(l_Lean_instInhabitedStructureParentInfo___closed__1); +l_Lean_instInhabitedStructureParentInfo = _init_l_Lean_instInhabitedStructureParentInfo(); +lean_mark_persistent(l_Lean_instInhabitedStructureParentInfo); l_Lean_instInhabitedStructureInfo___closed__1 = _init_l_Lean_instInhabitedStructureInfo___closed__1(); lean_mark_persistent(l_Lean_instInhabitedStructureInfo___closed__1); l_Lean_instInhabitedStructureInfo___closed__2 = _init_l_Lean_instInhabitedStructureInfo___closed__2(); @@ -4148,27 +4257,27 @@ l_Lean_instInhabitedStructureState___closed__2 = _init_l_Lean_instInhabitedStruc lean_mark_persistent(l_Lean_instInhabitedStructureState___closed__2); l_Lean_instInhabitedStructureState = _init_l_Lean_instInhabitedStructureState(); lean_mark_persistent(l_Lean_instInhabitedStructureState); -l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__2___closed__1 = _init_l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__2___closed__1(); -l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__2___closed__2 = _init_l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__2___closed__2(); -l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__2___closed__3 = _init_l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__2___closed__3(); -lean_mark_persistent(l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__2___closed__3); -l_Array_qsort_sort___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__5___closed__1 = _init_l_Array_qsort_sort___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__5___closed__1(); -lean_mark_persistent(l_Array_qsort_sort___at_Lean_initFn____x40_Lean_Structure___hyg_351____spec__5___closed__1); -l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__1 = _init_l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__1(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__1); -l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__2 = _init_l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__2(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__2); -l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__3 = _init_l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__3(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__3); -l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__4 = _init_l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__4(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__4); -l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__5 = _init_l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__5(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__5); -l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__6 = _init_l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__6(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__6); -l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__7 = _init_l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__7(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Structure___hyg_351____closed__7); -if (builtin) {res = l_Lean_initFn____x40_Lean_Structure___hyg_351_(lean_io_mk_world()); +l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__2___closed__1 = _init_l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__2___closed__1(); +l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__2___closed__2 = _init_l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__2___closed__2(); +l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__2___closed__3 = _init_l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__2___closed__3(); +lean_mark_persistent(l_Lean_PersistentHashMap_insertAux___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__2___closed__3); +l_Array_qsort_sort___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__5___closed__1 = _init_l_Array_qsort_sort___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__5___closed__1(); +lean_mark_persistent(l_Array_qsort_sort___at_Lean_initFn____x40_Lean_Structure___hyg_407____spec__5___closed__1); +l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__1 = _init_l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__1(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__1); +l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__2 = _init_l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__2(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__2); +l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__3 = _init_l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__3(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__3); +l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__4 = _init_l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__4(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__4); +l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__5 = _init_l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__5(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__5); +l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__6 = _init_l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__6(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__6); +l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__7 = _init_l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__7(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Structure___hyg_407____closed__7); +if (builtin) {res = l_Lean_initFn____x40_Lean_Structure___hyg_407_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_structureExt = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_structureExt); @@ -4181,10 +4290,18 @@ l_Array_qsort_sort___at_Lean_registerStructure___spec__2___closed__1 = _init_l_A lean_mark_persistent(l_Array_qsort_sort___at_Lean_registerStructure___spec__2___closed__1); l_Lean_registerStructure___closed__1 = _init_l_Lean_registerStructure___closed__1(); lean_mark_persistent(l_Lean_registerStructure___closed__1); +l_Lean_registerStructure___closed__2 = _init_l_Lean_registerStructure___closed__2(); +lean_mark_persistent(l_Lean_registerStructure___closed__2); +l_Lean_setStructureParents___rarg___lambda__2___closed__1 = _init_l_Lean_setStructureParents___rarg___lambda__2___closed__1(); +lean_mark_persistent(l_Lean_setStructureParents___rarg___lambda__2___closed__1); +l_Lean_setStructureParents___rarg___lambda__2___closed__2 = _init_l_Lean_setStructureParents___rarg___lambda__2___closed__2(); +lean_mark_persistent(l_Lean_setStructureParents___rarg___lambda__2___closed__2); +l_Lean_setStructureParents___rarg___lambda__2___closed__3 = _init_l_Lean_setStructureParents___rarg___lambda__2___closed__3(); +lean_mark_persistent(l_Lean_setStructureParents___rarg___lambda__2___closed__3); +l_Lean_setStructureParents___rarg___lambda__2___closed__4 = _init_l_Lean_setStructureParents___rarg___lambda__2___closed__4(); +lean_mark_persistent(l_Lean_setStructureParents___rarg___lambda__2___closed__4); l_Lean_getStructureInfo_x3f___closed__1 = _init_l_Lean_getStructureInfo_x3f___closed__1(); lean_mark_persistent(l_Lean_getStructureInfo_x3f___closed__1); -l_Lean_getStructureInfo_x3f___closed__2 = _init_l_Lean_getStructureInfo_x3f___closed__2(); -lean_mark_persistent(l_Lean_getStructureInfo_x3f___closed__2); l_Lean_getStructureCtor___closed__1 = _init_l_Lean_getStructureCtor___closed__1(); lean_mark_persistent(l_Lean_getStructureCtor___closed__1); l_Lean_getStructureCtor___closed__2 = _init_l_Lean_getStructureCtor___closed__2(); diff --git a/stage0/stdlib/Lean/SubExpr.c b/stage0/stdlib/Lean/SubExpr.c index 8a1d0ca291ed..100e41e89445 100644 --- a/stage0/stdlib/Lean/SubExpr.c +++ b/stage0/stdlib/Lean/SubExpr.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Lean.SubExpr -// Imports: Lean.Meta.Basic Lean.Data.Json Lean.Data.RBMap +// Imports: Lean.Meta.Basic Lean.Data.Json Lean.Data.RBMap Init.Control.Option #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -61,6 +61,7 @@ LEAN_EXPORT lean_object* l_Lean_SubExpr_Pos_foldr(lean_object*); extern lean_object* l_Lean_instInhabitedJson; static lean_object* l_Lean_SubExpr_instFromJsonGoalLocation___closed__1; LEAN_EXPORT lean_object* l_Lean_SubExpr_Pos_pushBindingBody___boxed(lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_SubExpr_instToJsonFVarId___lambda__1___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_SubExpr_Pos_tail___boxed(lean_object*); uint8_t lean_string_dec_eq(lean_object*, lean_object*); @@ -154,7 +155,6 @@ LEAN_EXPORT lean_object* l_Lean_SubExpr_Pos_pushAppFn___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_SubExpr_Pos_push(lean_object*, lean_object*); static lean_object* l___private_Lean_SubExpr_0__Lean_SubExpr_fromJsonGoalsLocation____x40_Lean_SubExpr___hyg_1812____closed__2; LEAN_EXPORT lean_object* l___private_Lean_SubExpr_0__Lean_SubExpr_fromJsonGoalLocation____x40_Lean_SubExpr___hyg_1411____lambda__3___boxed(lean_object*, lean_object*, lean_object*); -lean_object* l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_SubExpr_0__Lean_SubExpr_fromJsonGoalsLocation____x40_Lean_SubExpr___hyg_1812_(lean_object*); LEAN_EXPORT lean_object* l_Lean_SubExpr_Pos_asNat(lean_object*); static lean_object* l_Lean_SubExpr_Pos_typeCoord___closed__1; @@ -374,7 +374,7 @@ static lean_object* _init_l_Lean_SubExpr_Pos_head___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_SubExpr_Pos_head___closed__1; x_2 = l_Lean_SubExpr_Pos_head___closed__2; -x_3 = lean_unsigned_to_nat(43u); +x_3 = lean_unsigned_to_nat(44u); x_4 = lean_unsigned_to_nat(19u); x_5 = l_Lean_SubExpr_Pos_head___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -434,7 +434,7 @@ static lean_object* _init_l_Lean_SubExpr_Pos_tail___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_SubExpr_Pos_head___closed__1; x_2 = l_Lean_SubExpr_Pos_tail___closed__1; -x_3 = lean_unsigned_to_nat(47u); +x_3 = lean_unsigned_to_nat(48u); x_4 = lean_unsigned_to_nat(19u); x_5 = l_Lean_SubExpr_Pos_head___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -525,7 +525,7 @@ x_10 = l_Lean_SubExpr_Pos_push___closed__2; x_11 = lean_string_append(x_9, x_10); x_12 = l_Lean_SubExpr_Pos_head___closed__1; x_13 = l_Lean_SubExpr_Pos_push___closed__3; -x_14 = lean_unsigned_to_nat(51u); +x_14 = lean_unsigned_to_nat(52u); x_15 = lean_unsigned_to_nat(27u); x_16 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_12, x_13, x_14, x_15, x_11); lean_dec(x_11); @@ -1846,7 +1846,7 @@ lean_inc(x_3); lean_dec(x_2); x_4 = l_Lean_SubExpr_Pos_head___closed__1; x_5 = l_Lean_SubExpr_Pos_fromString_x21___closed__1; -x_6 = lean_unsigned_to_nat(139u); +x_6 = lean_unsigned_to_nat(140u); x_7 = lean_unsigned_to_nat(16u); x_8 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_4, x_5, x_6, x_7, x_3); lean_dec(x_3); @@ -2143,7 +2143,7 @@ static lean_object* _init_l_Lean_SubExpr_bindingBody_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_SubExpr_Pos_head___closed__1; x_2 = l_Lean_SubExpr_bindingBody_x21___closed__1; -x_3 = lean_unsigned_to_nat(178u); +x_3 = lean_unsigned_to_nat(179u); x_4 = lean_unsigned_to_nat(9u); x_5 = l_Lean_SubExpr_bindingBody_x21___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -2259,7 +2259,7 @@ static lean_object* _init_l_Lean_SubExpr_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_SubExpr_Pos_head___closed__1; x_2 = l_Lean_SubExpr_bindingDomain_x21___closed__1; -x_3 = lean_unsigned_to_nat(183u); +x_3 = lean_unsigned_to_nat(184u); x_4 = lean_unsigned_to_nat(9u); x_5 = l_Lean_SubExpr_bindingBody_x21___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -4783,7 +4783,7 @@ x_17 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_17, 0, x_10); lean_ctor_set(x_17, 1, x_16); x_18 = l_Lean_SubExpr_Pos_toArray___closed__2; -x_19 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_17, x_18); +x_19 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_17, x_18); x_20 = l_Lean_Json_mkObj(x_19); return x_20; } @@ -4878,6 +4878,7 @@ return x_5; lean_object* initialize_Lean_Meta_Basic(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Data_Json(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Data_RBMap(uint8_t builtin, lean_object*); +lean_object* initialize_Init_Control_Option(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Lean_SubExpr(uint8_t builtin, lean_object* w) { lean_object * res; @@ -4892,6 +4893,9 @@ lean_dec_ref(res); res = initialize_Lean_Data_RBMap(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +res = initialize_Init_Control_Option(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_SubExpr_Pos_maxChildren = _init_l_Lean_SubExpr_Pos_maxChildren(); lean_mark_persistent(l_Lean_SubExpr_Pos_maxChildren); l_Lean_SubExpr_Pos_typeCoord___closed__1 = _init_l_Lean_SubExpr_Pos_typeCoord___closed__1(); diff --git a/stage0/stdlib/Lean/Util/FileSetupInfo.c b/stage0/stdlib/Lean/Util/FileSetupInfo.c index bdf8c3d2ab91..d1c943478d7c 100644 --- a/stage0/stdlib/Lean/Util/FileSetupInfo.c +++ b/stage0/stdlib/Lean/Util/FileSetupInfo.c @@ -42,12 +42,12 @@ LEAN_EXPORT lean_object* l_Lean_instToJsonFileSetupInfo; static lean_object* l___private_Lean_Util_FileSetupInfo_0__Lean_fromJsonFileSetupInfo____x40_Lean_Util_FileSetupInfo___hyg_26____closed__7; static lean_object* l___private_Lean_Util_FileSetupInfo_0__Lean_fromJsonFileSetupInfo____x40_Lean_Util_FileSetupInfo___hyg_26____closed__9; LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Util_FileSetupInfo_0__Lean_fromJsonFileSetupInfo____x40_Lean_Util_FileSetupInfo___hyg_26____spec__2___boxed(lean_object*, lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(lean_object*, lean_object*); static lean_object* l___private_Lean_Util_FileSetupInfo_0__Lean_toJsonFileSetupInfo____x40_Lean_Util_FileSetupInfo___hyg_132____closed__1; LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Util_FileSetupInfo_0__Lean_fromJsonFileSetupInfo____x40_Lean_Util_FileSetupInfo___hyg_26____spec__1(lean_object*, lean_object*); lean_object* l___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40_(lean_object*); lean_object* l_Lean_RBNode_fold___at_Lean_instToJsonLeanOptions___spec__1(lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); -lean_object* l_List_bindTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(lean_object*, lean_object*); static lean_object* l___private_Lean_Util_FileSetupInfo_0__Lean_fromJsonFileSetupInfo____x40_Lean_Util_FileSetupInfo___hyg_26____closed__16; static lean_object* l___private_Lean_Util_FileSetupInfo_0__Lean_fromJsonFileSetupInfo____x40_Lean_Util_FileSetupInfo___hyg_26____closed__15; static lean_object* l___private_Lean_Util_FileSetupInfo_0__Lean_fromJsonFileSetupInfo____x40_Lean_Util_FileSetupInfo___hyg_26____closed__18; @@ -516,7 +516,7 @@ x_16 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_16, 0, x_7); lean_ctor_set(x_16, 1, x_15); x_17 = l___private_Lean_Util_FileSetupInfo_0__Lean_toJsonFileSetupInfo____x40_Lean_Util_FileSetupInfo___hyg_132____closed__1; -x_18 = l_List_bindTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(x_16, x_17); +x_18 = l_List_flatMapTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(x_16, x_17); x_19 = l_Lean_Json_mkObj(x_18); return x_19; } diff --git a/stage0/stdlib/Lean/Util/Paths.c b/stage0/stdlib/Lean/Util/Paths.c index 74cc605db6c5..c0633e6c3e92 100644 --- a/stage0/stdlib/Lean/Util/Paths.c +++ b/stage0/stdlib/Lean/Util/Paths.c @@ -52,6 +52,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Util_Paths_0__Lean_fromJsonLeanPaths__ static lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Util_Paths_0__Lean_fromJsonLeanPaths____x40_Lean_Util_Paths___hyg_106____spec__1___closed__1; LEAN_EXPORT uint8_t l___private_Lean_Util_Paths_0__Lean_fromJsonLeanPaths____x40_Lean_Util_Paths___hyg_106____lambda__1(lean_object*); static lean_object* l_Lean_initSrcSearchPath___closed__4; +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Paths_0__Lean_fromJsonLeanPaths____x40_Lean_Util_Paths___hyg_106____closed__12; LEAN_EXPORT lean_object* l_Lean_instToJsonLeanPaths; static lean_object* l___private_Lean_Util_Paths_0__Lean_fromJsonLeanPaths____x40_Lean_Util_Paths___hyg_106____closed__15; @@ -60,7 +61,6 @@ static lean_object* l___private_Lean_Util_Paths_0__Lean_fromJsonLeanPaths____x40 LEAN_EXPORT lean_object* l___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40_(lean_object*); lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____closed__2; -LEAN_EXPORT lean_object* l_List_bindTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Paths_0__Lean_fromJsonLeanPaths____x40_Lean_Util_Paths___hyg_106____closed__18; static lean_object* l___private_Lean_Util_Paths_0__Lean_fromJsonLeanPaths____x40_Lean_Util_Paths___hyg_106____closed__17; static lean_object* l___private_Lean_Util_Paths_0__Lean_fromJsonLeanPaths____x40_Lean_Util_Paths___hyg_106____closed__9; @@ -109,7 +109,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_List_bindTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -224,7 +224,7 @@ x_29 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_29, 0, x_13); lean_ctor_set(x_29, 1, x_28); x_30 = l___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____closed__4; -x_31 = l_List_bindTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(x_29, x_30); +x_31 = l_List_flatMapTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(x_29, x_30); x_32 = l_Lean_Json_mkObj(x_31); return x_32; } diff --git a/stage0/stdlib/Lean/Util/Profiler.c b/stage0/stdlib/Lean/Util/Profiler.c index f4befe5f2bb0..5e9b5cad6ba3 100644 --- a/stage0/stdlib/Lean/Util/Profiler.c +++ b/stage0/stdlib/Lean/Util/Profiler.c @@ -161,6 +161,7 @@ static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonStack LEAN_EXPORT lean_object* l_Lean_Firefox_instFromJsonThread; static lean_object* l_Lean_Firefox_instFromJsonCategory___closed__1; LEAN_EXPORT lean_object* l_Lean_Firefox_Profile_collide(lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfile____x40_Lean_Util_Profiler___hyg_3535____closed__14; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonSamplesTable____x40_Lean_Util_Profiler___hyg_1172____closed__3; LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfile____x40_Lean_Util_Profiler___hyg_3535____spec__2___boxed(lean_object*, lean_object*); @@ -403,7 +404,6 @@ static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFuncT LEAN_EXPORT uint8_t l___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Firefox_instFromJsonProfile; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFuncTable____x40_Lean_Util_Profiler___hyg_1585____closed__1; -lean_object* l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonProfileMeta____x40_Lean_Util_Profiler___hyg_634_(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonRawMarkerTable____x40_Lean_Util_Profiler___hyg_2419_(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__30(uint8_t, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); @@ -1323,7 +1323,7 @@ x_23 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_23, 0, x_9); lean_ctor_set(x_23, 1, x_22); x_24 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_25 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_23, x_24); +x_25 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_23, x_24); x_26 = l_Lean_Json_mkObj(x_25); return x_26; } @@ -2751,7 +2751,7 @@ x_53 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_53, 0, x_47); lean_ctor_set(x_53, 1, x_52); x_54 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_55 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_53, x_54); +x_55 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_53, x_54); x_56 = l_Lean_Json_mkObj(x_55); return x_56; } @@ -2777,7 +2777,7 @@ x_63 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_63, 0, x_47); lean_ctor_set(x_63, 1, x_62); x_64 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_65 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_63, x_64); +x_65 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_63, x_64); x_66 = l_Lean_Json_mkObj(x_65); return x_66; } @@ -2804,7 +2804,7 @@ x_72 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_72, 0, x_47); lean_ctor_set(x_72, 1, x_71); x_73 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_74 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_72, x_73); +x_74 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_72, x_73); x_75 = l_Lean_Json_mkObj(x_74); return x_75; } @@ -2830,7 +2830,7 @@ x_82 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_82, 0, x_47); lean_ctor_set(x_82, 1, x_81); x_83 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_84 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_82, x_83); +x_84 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_82, x_83); x_85 = l_Lean_Json_mkObj(x_84); return x_85; } @@ -2884,7 +2884,7 @@ x_98 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_98, 0, x_90); lean_ctor_set(x_98, 1, x_97); x_99 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_100 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_98, x_99); +x_100 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_98, x_99); x_101 = l_Lean_Json_mkObj(x_100); return x_101; } @@ -2921,7 +2921,7 @@ x_109 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_109, 0, x_90); lean_ctor_set(x_109, 1, x_108); x_110 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_111 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_109, x_110); +x_111 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_109, x_110); x_112 = l_Lean_Json_mkObj(x_111); return x_112; } @@ -2964,7 +2964,7 @@ x_122 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_122, 0, x_116); lean_ctor_set(x_122, 1, x_121); x_123 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_124 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_122, x_123); +x_124 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_122, x_123); x_125 = l_Lean_Json_mkObj(x_124); return x_125; } @@ -2990,7 +2990,7 @@ x_132 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_132, 0, x_116); lean_ctor_set(x_132, 1, x_131); x_133 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_134 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_132, x_133); +x_134 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_132, x_133); x_135 = l_Lean_Json_mkObj(x_134); return x_135; } @@ -3017,7 +3017,7 @@ x_141 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_141, 0, x_116); lean_ctor_set(x_141, 1, x_140); x_142 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_143 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_141, x_142); +x_143 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_141, x_142); x_144 = l_Lean_Json_mkObj(x_143); return x_144; } @@ -3043,7 +3043,7 @@ x_151 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_151, 0, x_116); lean_ctor_set(x_151, 1, x_150); x_152 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_153 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_151, x_152); +x_153 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_151, x_152); x_154 = l_Lean_Json_mkObj(x_153); return x_154; } @@ -3097,7 +3097,7 @@ x_167 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_167, 0, x_159); lean_ctor_set(x_167, 1, x_166); x_168 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_169 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_167, x_168); +x_169 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_167, x_168); x_170 = l_Lean_Json_mkObj(x_169); return x_170; } @@ -3134,7 +3134,7 @@ x_178 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_178, 0, x_159); lean_ctor_set(x_178, 1, x_177); x_179 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_180 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_178, x_179); +x_180 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_178, x_179); x_181 = l_Lean_Json_mkObj(x_180); return x_181; } @@ -4301,7 +4301,7 @@ x_42 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_42, 0, x_10); lean_ctor_set(x_42, 1, x_41); x_43 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_44 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_42, x_43); +x_44 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_42, x_43); x_45 = l_Lean_Json_mkObj(x_44); return x_45; } @@ -5224,7 +5224,7 @@ x_40 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_40, 0, x_10); lean_ctor_set(x_40, 1, x_39); x_41 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_42 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_40, x_41); +x_42 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_40, x_41); x_43 = l_Lean_Json_mkObj(x_42); return x_43; } @@ -6347,7 +6347,7 @@ x_66 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_66, 0, x_10); lean_ctor_set(x_66, 1, x_65); x_67 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_68 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_66, x_67); +x_68 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_66, x_67); x_69 = l_Lean_Json_mkObj(x_68); return x_69; } @@ -6865,7 +6865,7 @@ x_34 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_34, 0, x_10); lean_ctor_set(x_34, 1, x_33); x_35 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_36 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_34, x_35); +x_36 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_34, x_35); x_37 = l_Lean_Json_mkObj(x_36); return x_37; } @@ -7233,7 +7233,7 @@ x_26 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_26, 0, x_10); lean_ctor_set(x_26, 1, x_25); x_27 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_28 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_26, x_27); +x_28 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_26, x_27); x_29 = l_Lean_Json_mkObj(x_28); return x_29; } @@ -7522,7 +7522,7 @@ x_18 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_18, 0, x_10); lean_ctor_set(x_18, 1, x_17); x_19 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_20 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_18, x_19); +x_20 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_18, x_19); x_21 = l_Lean_Json_mkObj(x_20); return x_21; } @@ -8762,7 +8762,7 @@ x_65 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_65, 0, x_16); lean_ctor_set(x_65, 1, x_64); x_66 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_67 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_65, x_66); +x_67 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_65, x_66); x_68 = l_Lean_Json_mkObj(x_67); return x_68; } @@ -9388,7 +9388,7 @@ x_25 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_25, 0, x_7); lean_ctor_set(x_25, 1, x_24); x_26 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_27 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_25, x_26); +x_27 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_25, x_26); x_28 = l_Lean_Json_mkObj(x_27); return x_28; } diff --git a/stage0/stdlib/Lean/Util/Recognizers.c b/stage0/stdlib/Lean/Util/Recognizers.c index 98c038c5e35c..06b430b9fbf2 100644 --- a/stage0/stdlib/Lean/Util/Recognizers.c +++ b/stage0/stdlib/Lean/Util/Recognizers.c @@ -13,22 +13,29 @@ #ifdef __cplusplus extern "C" { #endif +lean_object* l_Lean_Expr_rawNatLit_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_and_x3f(lean_object*); static lean_object* l_Lean_Expr_natAdd_x3f___closed__2; +static lean_object* l_Lean_Expr_name_x3f___closed__1; static lean_object* l_Lean_Expr_heq_x3f___closed__2; static lean_object* l_Lean_Expr_listLit_x3f_loop___closed__1; LEAN_EXPORT uint8_t l_Lean_Expr_isDIte(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_arrow_x3f___boxed(lean_object*); static lean_object* l_Lean_Expr_not_x3f___closed__2; +static lean_object* l_Lean_Expr_name_x3f___closed__6; static lean_object* l_Lean_Expr_eq_x3f___closed__1; +LEAN_EXPORT lean_object* l_Lean_Expr_name_x3f(lean_object*); static lean_object* l_Lean_Expr_arrayLit_x3f___closed__1; LEAN_EXPORT lean_object* l_Lean_Expr_isHEq___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_app1_x3f(lean_object*, lean_object*); uint8_t l_Lean_Expr_isAppOfArity(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_natAdd_x3f___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_not_x3f___boxed(lean_object*); +static lean_object* l_Lean_Expr_name_x3f___closed__10; +static lean_object* l_Lean_Expr_name_x3f___closed__11; LEAN_EXPORT lean_object* l_Lean_Expr_eq_x3f___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_notNot_x3f(lean_object*); +static lean_object* l_Lean_Expr_name_x3f___closed__2; LEAN_EXPORT lean_object* l_Lean_Expr_not_x3f(lean_object*); static lean_object* l_Lean_Expr_isIte___closed__2; static lean_object* l_Lean_Expr_prod_x3f___closed__1; @@ -38,24 +45,33 @@ LEAN_EXPORT lean_object* l_Lean_Expr_arrayLit_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_ne_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_app3_x3f(lean_object*, lean_object*); static lean_object* l_Lean_Expr_and_x3f___closed__2; +lean_object* l_Lean_Name_mkStr5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_appFn_x21_x27(lean_object*); +uint8_t lean_string_dec_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_ne_x3f___boxed(lean_object*); lean_object* l_Lean_Expr_appArg_x21(lean_object*); static lean_object* l_Lean_Expr_arrayLit_x3f___closed__2; LEAN_EXPORT lean_object* l_Lean_Expr_app4_x3f___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Expr_name_x3f___closed__7; +lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_natAdd_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_eqOrIff_x3f(lean_object*); +static lean_object* l_Lean_Expr_name_x3f___closed__3; uint8_t l_Lean_Expr_isAppOfArity_x27(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_const_x3f(lean_object*); +lean_object* l_Lean_Name_mkStr7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_and_x3f___boxed(lean_object*); static lean_object* l_Lean_Expr_heq_x3f___closed__1; LEAN_EXPORT lean_object* l_Lean_Expr_iff_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_isEq___boxed(lean_object*); static lean_object* l_Lean_Expr_listLit_x3f_loop___closed__2; LEAN_EXPORT uint8_t l_Lean_Expr_isEq(lean_object*); +static lean_object* l_Lean_Expr_name_x3f___closed__8; LEAN_EXPORT lean_object* l_Lean_Expr_arrow_x3f(lean_object*); +static lean_object* l_Lean_Expr_name_x3f___closed__5; uint8_t l_Lean_Expr_hasLooseBVars(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_listLit_x3f(lean_object*); +lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_prod_x3f(lean_object*); static lean_object* l_Lean_Expr_and_x3f___closed__1; static lean_object* l_Lean_Expr_natAdd_x3f___closed__1; @@ -64,16 +80,20 @@ LEAN_EXPORT lean_object* l_Lean_Expr_listLit_x3f_loop(lean_object*, lean_object* static lean_object* l_Lean_Expr_ne_x3f___closed__1; LEAN_EXPORT lean_object* l_Lean_Expr_isDIte___boxed(lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); +static lean_object* l_Lean_Expr_name_x3f___closed__12; static lean_object* l_Lean_Expr_isDIte___closed__1; LEAN_EXPORT lean_object* l_Lean_Expr_app2_x3f(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Expr_isIte(lean_object*); static lean_object* l_Lean_Expr_listLit_x3f_loop___closed__3; lean_object* l_Lean_Expr_appFn_x21(lean_object*); +static lean_object* l_Lean_Expr_name_x3f___closed__14; LEAN_EXPORT lean_object* l_Lean_Expr_eqOrIff_x3f___boxed(lean_object*); +lean_object* l_Lean_Name_mkStr6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Expr_isDIte___closed__2; LEAN_EXPORT lean_object* l_Lean_Expr_arrayLit_x3f___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_app1_x3f___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Expr_natAdd_x3f___closed__3; +static lean_object* l_Lean_Expr_name_x3f___closed__9; static lean_object* l_Lean_Expr_iff_x3f___closed__1; LEAN_EXPORT lean_object* l_Lean_Expr_eq_x3f(lean_object*); lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); @@ -82,6 +102,7 @@ LEAN_EXPORT uint8_t l_Lean_Expr_isHEq(lean_object*); static lean_object* l_Lean_Expr_listLit_x3f_loop___closed__4; LEAN_EXPORT lean_object* l_Lean_Expr_app4_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_iff_x3f___boxed(lean_object*); +static lean_object* l_Lean_Expr_name_x3f___closed__4; LEAN_EXPORT lean_object* l_Lean_Expr_heq_x3f___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_prod_x3f___boxed(lean_object*); lean_object* l_List_reverse___rarg(lean_object*); @@ -89,12 +110,16 @@ LEAN_EXPORT lean_object* l_Lean_Expr_isIte___boxed(lean_object*); lean_object* l_Lean_Expr_appArg_x21_x27(lean_object*); static lean_object* l_Lean_Expr_iff_x3f___closed__2; static lean_object* l_Lean_Expr_prod_x3f___closed__2; +lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_heq_x3f(lean_object*); static lean_object* l_Lean_Expr_eq_x3f___closed__2; +static lean_object* l_Lean_Expr_name_x3f___closed__13; LEAN_EXPORT lean_object* l_Lean_Expr_notNot_x3f___boxed(lean_object*); +lean_object* l_Lean_Expr_nat_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_app3_x3f___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Expr_isIte___closed__1; LEAN_EXPORT lean_object* l_Lean_Expr_app2_x3f___boxed(lean_object*, lean_object*); +lean_object* l_Lean_Name_mkStr8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_const_x3f(lean_object* x_1) { _start: { @@ -1187,6 +1212,3298 @@ lean_dec(x_1); return x_2; } } +static lean_object* _init_l_Lean_Expr_name_x3f___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Expr_name_x3f___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Name", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Expr_name_x3f___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("anonymous", 9, 9); +return x_1; +} +} +static lean_object* _init_l_Lean_Expr_name_x3f___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Expr_name_x3f___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mkStr1", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_Expr_name_x3f___closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("str", 3, 3); +return x_1; +} +} +static lean_object* _init_l_Lean_Expr_name_x3f___closed__7() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("num", 3, 3); +return x_1; +} +} +static lean_object* _init_l_Lean_Expr_name_x3f___closed__8() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mkStr2", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_Expr_name_x3f___closed__9() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mkStr3", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_Expr_name_x3f___closed__10() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mkStr4", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_Expr_name_x3f___closed__11() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mkStr5", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_Expr_name_x3f___closed__12() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mkStr6", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_Expr_name_x3f___closed__13() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mkStr7", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_Expr_name_x3f___closed__14() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mkStr8", 6, 6); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Expr_name_x3f(lean_object* x_1) { +_start: +{ +switch (lean_obj_tag(x_1)) { +case 4: +{ +lean_object* x_2; +x_2 = lean_ctor_get(x_1, 0); +lean_inc(x_2); +lean_dec(x_1); +if (lean_obj_tag(x_2) == 1) +{ +lean_object* x_3; +x_3 = lean_ctor_get(x_2, 0); +lean_inc(x_3); +if (lean_obj_tag(x_3) == 1) +{ +lean_object* x_4; +x_4 = lean_ctor_get(x_3, 0); +lean_inc(x_4); +if (lean_obj_tag(x_4) == 1) +{ +lean_object* x_5; +x_5 = lean_ctor_get(x_4, 0); +lean_inc(x_5); +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; +x_6 = lean_ctor_get(x_2, 1); +lean_inc(x_6); +lean_dec(x_2); +x_7 = lean_ctor_get(x_3, 1); +lean_inc(x_7); +lean_dec(x_3); +x_8 = lean_ctor_get(x_4, 1); +lean_inc(x_8); +lean_dec(x_4); +x_9 = l_Lean_Expr_name_x3f___closed__1; +x_10 = lean_string_dec_eq(x_8, x_9); +lean_dec(x_8); +if (x_10 == 0) +{ +lean_object* x_11; +lean_dec(x_7); +lean_dec(x_6); +x_11 = lean_box(0); +return x_11; +} +else +{ +lean_object* x_12; uint8_t x_13; +x_12 = l_Lean_Expr_name_x3f___closed__2; +x_13 = lean_string_dec_eq(x_7, x_12); +lean_dec(x_7); +if (x_13 == 0) +{ +lean_object* x_14; +lean_dec(x_6); +x_14 = lean_box(0); +return x_14; +} +else +{ +lean_object* x_15; uint8_t x_16; +x_15 = l_Lean_Expr_name_x3f___closed__3; +x_16 = lean_string_dec_eq(x_6, x_15); +lean_dec(x_6); +if (x_16 == 0) +{ +lean_object* x_17; +x_17 = lean_box(0); +return x_17; +} +else +{ +lean_object* x_18; +x_18 = l_Lean_Expr_name_x3f___closed__4; +return x_18; +} +} +} +} +else +{ +lean_object* x_19; +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_19 = lean_box(0); +return x_19; +} +} +else +{ +lean_object* x_20; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_20 = lean_box(0); +return x_20; +} +} +else +{ +lean_object* x_21; +lean_dec(x_3); +lean_dec(x_2); +x_21 = lean_box(0); +return x_21; +} +} +else +{ +lean_object* x_22; +lean_dec(x_2); +x_22 = lean_box(0); +return x_22; +} +} +case 5: +{ +lean_object* x_23; +x_23 = lean_ctor_get(x_1, 0); +lean_inc(x_23); +switch (lean_obj_tag(x_23)) { +case 4: +{ +lean_object* x_24; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +lean_dec(x_23); +if (lean_obj_tag(x_24) == 1) +{ +lean_object* x_25; +x_25 = lean_ctor_get(x_24, 0); +lean_inc(x_25); +if (lean_obj_tag(x_25) == 1) +{ +lean_object* x_26; +x_26 = lean_ctor_get(x_25, 0); +lean_inc(x_26); +if (lean_obj_tag(x_26) == 1) +{ +lean_object* x_27; +x_27 = lean_ctor_get(x_26, 0); +lean_inc(x_27); +if (lean_obj_tag(x_27) == 0) +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +lean_dec(x_1); +x_29 = lean_ctor_get(x_24, 1); +lean_inc(x_29); +lean_dec(x_24); +x_30 = lean_ctor_get(x_25, 1); +lean_inc(x_30); +lean_dec(x_25); +x_31 = lean_ctor_get(x_26, 1); +lean_inc(x_31); +lean_dec(x_26); +x_32 = l_Lean_Expr_name_x3f___closed__1; +x_33 = lean_string_dec_eq(x_31, x_32); +lean_dec(x_31); +if (x_33 == 0) +{ +lean_object* x_34; +lean_dec(x_30); +lean_dec(x_29); +lean_dec(x_28); +x_34 = lean_box(0); +return x_34; +} +else +{ +lean_object* x_35; uint8_t x_36; +x_35 = l_Lean_Expr_name_x3f___closed__2; +x_36 = lean_string_dec_eq(x_30, x_35); +lean_dec(x_30); +if (x_36 == 0) +{ +lean_object* x_37; +lean_dec(x_29); +lean_dec(x_28); +x_37 = lean_box(0); +return x_37; +} +else +{ +lean_object* x_38; uint8_t x_39; +x_38 = l_Lean_Expr_name_x3f___closed__5; +x_39 = lean_string_dec_eq(x_29, x_38); +lean_dec(x_29); +if (x_39 == 0) +{ +lean_object* x_40; +lean_dec(x_28); +x_40 = lean_box(0); +return x_40; +} +else +{ +if (lean_obj_tag(x_28) == 9) +{ +lean_object* x_41; +x_41 = lean_ctor_get(x_28, 0); +lean_inc(x_41); +lean_dec(x_28); +if (lean_obj_tag(x_41) == 0) +{ +lean_object* x_42; +lean_dec(x_41); +x_42 = lean_box(0); +return x_42; +} +else +{ +uint8_t x_43; +x_43 = !lean_is_exclusive(x_41); +if (x_43 == 0) +{ +lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_44 = lean_ctor_get(x_41, 0); +x_45 = lean_box(0); +x_46 = l_Lean_Name_str___override(x_45, x_44); +lean_ctor_set(x_41, 0, x_46); +return x_41; +} +else +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_47 = lean_ctor_get(x_41, 0); +lean_inc(x_47); +lean_dec(x_41); +x_48 = lean_box(0); +x_49 = l_Lean_Name_str___override(x_48, x_47); +x_50 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_50, 0, x_49); +return x_50; +} +} +} +else +{ +lean_object* x_51; +lean_dec(x_28); +x_51 = lean_box(0); +return x_51; +} +} +} +} +} +else +{ +lean_object* x_52; +lean_dec(x_27); +lean_dec(x_26); +lean_dec(x_25); +lean_dec(x_24); +lean_dec(x_1); +x_52 = lean_box(0); +return x_52; +} +} +else +{ +lean_object* x_53; +lean_dec(x_26); +lean_dec(x_25); +lean_dec(x_24); +lean_dec(x_1); +x_53 = lean_box(0); +return x_53; +} +} +else +{ +lean_object* x_54; +lean_dec(x_25); +lean_dec(x_24); +lean_dec(x_1); +x_54 = lean_box(0); +return x_54; +} +} +else +{ +lean_object* x_55; +lean_dec(x_24); +lean_dec(x_1); +x_55 = lean_box(0); +return x_55; +} +} +case 5: +{ +lean_object* x_56; +x_56 = lean_ctor_get(x_23, 0); +lean_inc(x_56); +switch (lean_obj_tag(x_56)) { +case 4: +{ +lean_object* x_57; +x_57 = lean_ctor_get(x_56, 0); +lean_inc(x_57); +lean_dec(x_56); +if (lean_obj_tag(x_57) == 1) +{ +lean_object* x_58; +x_58 = lean_ctor_get(x_57, 0); +lean_inc(x_58); +if (lean_obj_tag(x_58) == 1) +{ +lean_object* x_59; +x_59 = lean_ctor_get(x_58, 0); +lean_inc(x_59); +if (lean_obj_tag(x_59) == 1) +{ +lean_object* x_60; +x_60 = lean_ctor_get(x_59, 0); +lean_inc(x_60); +if (lean_obj_tag(x_60) == 0) +{ +lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; uint8_t x_67; +x_61 = lean_ctor_get(x_1, 1); +lean_inc(x_61); +lean_dec(x_1); +x_62 = lean_ctor_get(x_23, 1); +lean_inc(x_62); +lean_dec(x_23); +x_63 = lean_ctor_get(x_57, 1); +lean_inc(x_63); +lean_dec(x_57); +x_64 = lean_ctor_get(x_58, 1); +lean_inc(x_64); +lean_dec(x_58); +x_65 = lean_ctor_get(x_59, 1); +lean_inc(x_65); +lean_dec(x_59); +x_66 = l_Lean_Expr_name_x3f___closed__1; +x_67 = lean_string_dec_eq(x_65, x_66); +lean_dec(x_65); +if (x_67 == 0) +{ +lean_object* x_68; +lean_dec(x_64); +lean_dec(x_63); +lean_dec(x_62); +lean_dec(x_61); +x_68 = lean_box(0); +return x_68; +} +else +{ +lean_object* x_69; uint8_t x_70; +x_69 = l_Lean_Expr_name_x3f___closed__2; +x_70 = lean_string_dec_eq(x_64, x_69); +lean_dec(x_64); +if (x_70 == 0) +{ +lean_object* x_71; +lean_dec(x_63); +lean_dec(x_62); +lean_dec(x_61); +x_71 = lean_box(0); +return x_71; +} +else +{ +lean_object* x_72; uint8_t x_73; +x_72 = l_Lean_Expr_name_x3f___closed__6; +x_73 = lean_string_dec_eq(x_63, x_72); +if (x_73 == 0) +{ +lean_object* x_74; uint8_t x_75; +x_74 = l_Lean_Expr_name_x3f___closed__7; +x_75 = lean_string_dec_eq(x_63, x_74); +if (x_75 == 0) +{ +lean_object* x_76; uint8_t x_77; +x_76 = l_Lean_Expr_name_x3f___closed__8; +x_77 = lean_string_dec_eq(x_63, x_76); +lean_dec(x_63); +if (x_77 == 0) +{ +lean_object* x_78; +lean_dec(x_62); +lean_dec(x_61); +x_78 = lean_box(0); +return x_78; +} +else +{ +if (lean_obj_tag(x_62) == 9) +{ +lean_object* x_79; +x_79 = lean_ctor_get(x_62, 0); +lean_inc(x_79); +lean_dec(x_62); +if (lean_obj_tag(x_79) == 0) +{ +lean_object* x_80; +lean_dec(x_79); +lean_dec(x_61); +x_80 = lean_box(0); +return x_80; +} +else +{ +if (lean_obj_tag(x_61) == 9) +{ +lean_object* x_81; +x_81 = lean_ctor_get(x_61, 0); +lean_inc(x_81); +lean_dec(x_61); +if (lean_obj_tag(x_81) == 0) +{ +lean_object* x_82; +lean_dec(x_81); +lean_dec(x_79); +x_82 = lean_box(0); +return x_82; +} +else +{ +lean_object* x_83; uint8_t x_84; +x_83 = lean_ctor_get(x_79, 0); +lean_inc(x_83); +lean_dec(x_79); +x_84 = !lean_is_exclusive(x_81); +if (x_84 == 0) +{ +lean_object* x_85; lean_object* x_86; +x_85 = lean_ctor_get(x_81, 0); +x_86 = l_Lean_Name_mkStr2(x_83, x_85); +lean_ctor_set(x_81, 0, x_86); +return x_81; +} +else +{ +lean_object* x_87; lean_object* x_88; lean_object* x_89; +x_87 = lean_ctor_get(x_81, 0); +lean_inc(x_87); +lean_dec(x_81); +x_88 = l_Lean_Name_mkStr2(x_83, x_87); +x_89 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_89, 0, x_88); +return x_89; +} +} +} +else +{ +lean_object* x_90; +lean_dec(x_79); +lean_dec(x_61); +x_90 = lean_box(0); +return x_90; +} +} +} +else +{ +lean_object* x_91; +lean_dec(x_62); +lean_dec(x_61); +x_91 = lean_box(0); +return x_91; +} +} +} +else +{ +lean_object* x_92; +lean_dec(x_63); +lean_inc(x_61); +x_92 = l_Lean_Expr_rawNatLit_x3f(x_61); +if (lean_obj_tag(x_92) == 0) +{ +lean_object* x_93; +x_93 = l_Lean_Expr_nat_x3f(x_61); +if (lean_obj_tag(x_93) == 0) +{ +lean_object* x_94; +lean_dec(x_62); +x_94 = lean_box(0); +return x_94; +} +else +{ +lean_object* x_95; lean_object* x_96; +x_95 = lean_ctor_get(x_93, 0); +lean_inc(x_95); +lean_dec(x_93); +x_96 = l_Lean_Expr_name_x3f(x_62); +if (lean_obj_tag(x_96) == 0) +{ +lean_object* x_97; +lean_dec(x_95); +x_97 = lean_box(0); +return x_97; +} +else +{ +uint8_t x_98; +x_98 = !lean_is_exclusive(x_96); +if (x_98 == 0) +{ +lean_object* x_99; lean_object* x_100; +x_99 = lean_ctor_get(x_96, 0); +x_100 = l_Lean_Name_num___override(x_99, x_95); +lean_ctor_set(x_96, 0, x_100); +return x_96; +} +else +{ +lean_object* x_101; lean_object* x_102; lean_object* x_103; +x_101 = lean_ctor_get(x_96, 0); +lean_inc(x_101); +lean_dec(x_96); +x_102 = l_Lean_Name_num___override(x_101, x_95); +x_103 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_103, 0, x_102); +return x_103; +} +} +} +} +else +{ +lean_object* x_104; lean_object* x_105; +lean_dec(x_61); +x_104 = lean_ctor_get(x_92, 0); +lean_inc(x_104); +lean_dec(x_92); +x_105 = l_Lean_Expr_name_x3f(x_62); +if (lean_obj_tag(x_105) == 0) +{ +lean_object* x_106; +lean_dec(x_104); +x_106 = lean_box(0); +return x_106; +} +else +{ +uint8_t x_107; +x_107 = !lean_is_exclusive(x_105); +if (x_107 == 0) +{ +lean_object* x_108; lean_object* x_109; +x_108 = lean_ctor_get(x_105, 0); +x_109 = l_Lean_Name_num___override(x_108, x_104); +lean_ctor_set(x_105, 0, x_109); +return x_105; +} +else +{ +lean_object* x_110; lean_object* x_111; lean_object* x_112; +x_110 = lean_ctor_get(x_105, 0); +lean_inc(x_110); +lean_dec(x_105); +x_111 = l_Lean_Name_num___override(x_110, x_104); +x_112 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_112, 0, x_111); +return x_112; +} +} +} +} +} +else +{ +lean_dec(x_63); +if (lean_obj_tag(x_61) == 9) +{ +lean_object* x_113; +x_113 = lean_ctor_get(x_61, 0); +lean_inc(x_113); +lean_dec(x_61); +if (lean_obj_tag(x_113) == 0) +{ +lean_object* x_114; +lean_dec(x_113); +lean_dec(x_62); +x_114 = lean_box(0); +return x_114; +} +else +{ +lean_object* x_115; lean_object* x_116; +x_115 = lean_ctor_get(x_113, 0); +lean_inc(x_115); +lean_dec(x_113); +x_116 = l_Lean_Expr_name_x3f(x_62); +if (lean_obj_tag(x_116) == 0) +{ +lean_object* x_117; +lean_dec(x_115); +x_117 = lean_box(0); +return x_117; +} +else +{ +uint8_t x_118; +x_118 = !lean_is_exclusive(x_116); +if (x_118 == 0) +{ +lean_object* x_119; lean_object* x_120; +x_119 = lean_ctor_get(x_116, 0); +x_120 = l_Lean_Name_str___override(x_119, x_115); +lean_ctor_set(x_116, 0, x_120); +return x_116; +} +else +{ +lean_object* x_121; lean_object* x_122; lean_object* x_123; +x_121 = lean_ctor_get(x_116, 0); +lean_inc(x_121); +lean_dec(x_116); +x_122 = l_Lean_Name_str___override(x_121, x_115); +x_123 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_123, 0, x_122); +return x_123; +} +} +} +} +else +{ +lean_object* x_124; +lean_dec(x_62); +lean_dec(x_61); +x_124 = lean_box(0); +return x_124; +} +} +} +} +} +else +{ +lean_object* x_125; +lean_dec(x_60); +lean_dec(x_59); +lean_dec(x_58); +lean_dec(x_57); +lean_dec(x_23); +lean_dec(x_1); +x_125 = lean_box(0); +return x_125; +} +} +else +{ +lean_object* x_126; +lean_dec(x_59); +lean_dec(x_58); +lean_dec(x_57); +lean_dec(x_23); +lean_dec(x_1); +x_126 = lean_box(0); +return x_126; +} +} +else +{ +lean_object* x_127; +lean_dec(x_58); +lean_dec(x_57); +lean_dec(x_23); +lean_dec(x_1); +x_127 = lean_box(0); +return x_127; +} +} +else +{ +lean_object* x_128; +lean_dec(x_57); +lean_dec(x_23); +lean_dec(x_1); +x_128 = lean_box(0); +return x_128; +} +} +case 5: +{ +lean_object* x_129; +x_129 = lean_ctor_get(x_56, 0); +lean_inc(x_129); +switch (lean_obj_tag(x_129)) { +case 4: +{ +lean_object* x_130; +x_130 = lean_ctor_get(x_129, 0); +lean_inc(x_130); +lean_dec(x_129); +if (lean_obj_tag(x_130) == 1) +{ +lean_object* x_131; +x_131 = lean_ctor_get(x_130, 0); +lean_inc(x_131); +if (lean_obj_tag(x_131) == 1) +{ +lean_object* x_132; +x_132 = lean_ctor_get(x_131, 0); +lean_inc(x_132); +if (lean_obj_tag(x_132) == 1) +{ +lean_object* x_133; +x_133 = lean_ctor_get(x_132, 0); +lean_inc(x_133); +if (lean_obj_tag(x_133) == 0) +{ +lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; uint8_t x_141; +x_134 = lean_ctor_get(x_1, 1); +lean_inc(x_134); +lean_dec(x_1); +x_135 = lean_ctor_get(x_23, 1); +lean_inc(x_135); +lean_dec(x_23); +x_136 = lean_ctor_get(x_56, 1); +lean_inc(x_136); +lean_dec(x_56); +x_137 = lean_ctor_get(x_130, 1); +lean_inc(x_137); +lean_dec(x_130); +x_138 = lean_ctor_get(x_131, 1); +lean_inc(x_138); +lean_dec(x_131); +x_139 = lean_ctor_get(x_132, 1); +lean_inc(x_139); +lean_dec(x_132); +x_140 = l_Lean_Expr_name_x3f___closed__1; +x_141 = lean_string_dec_eq(x_139, x_140); +lean_dec(x_139); +if (x_141 == 0) +{ +lean_object* x_142; +lean_dec(x_138); +lean_dec(x_137); +lean_dec(x_136); +lean_dec(x_135); +lean_dec(x_134); +x_142 = lean_box(0); +return x_142; +} +else +{ +lean_object* x_143; uint8_t x_144; +x_143 = l_Lean_Expr_name_x3f___closed__2; +x_144 = lean_string_dec_eq(x_138, x_143); +lean_dec(x_138); +if (x_144 == 0) +{ +lean_object* x_145; +lean_dec(x_137); +lean_dec(x_136); +lean_dec(x_135); +lean_dec(x_134); +x_145 = lean_box(0); +return x_145; +} +else +{ +lean_object* x_146; uint8_t x_147; +x_146 = l_Lean_Expr_name_x3f___closed__9; +x_147 = lean_string_dec_eq(x_137, x_146); +lean_dec(x_137); +if (x_147 == 0) +{ +lean_object* x_148; +lean_dec(x_136); +lean_dec(x_135); +lean_dec(x_134); +x_148 = lean_box(0); +return x_148; +} +else +{ +if (lean_obj_tag(x_136) == 9) +{ +lean_object* x_149; +x_149 = lean_ctor_get(x_136, 0); +lean_inc(x_149); +lean_dec(x_136); +if (lean_obj_tag(x_149) == 0) +{ +lean_object* x_150; +lean_dec(x_149); +lean_dec(x_135); +lean_dec(x_134); +x_150 = lean_box(0); +return x_150; +} +else +{ +if (lean_obj_tag(x_135) == 9) +{ +lean_object* x_151; +x_151 = lean_ctor_get(x_135, 0); +lean_inc(x_151); +lean_dec(x_135); +if (lean_obj_tag(x_151) == 0) +{ +lean_object* x_152; +lean_dec(x_151); +lean_dec(x_149); +lean_dec(x_134); +x_152 = lean_box(0); +return x_152; +} +else +{ +if (lean_obj_tag(x_134) == 9) +{ +lean_object* x_153; +x_153 = lean_ctor_get(x_134, 0); +lean_inc(x_153); +lean_dec(x_134); +if (lean_obj_tag(x_153) == 0) +{ +lean_object* x_154; +lean_dec(x_153); +lean_dec(x_151); +lean_dec(x_149); +x_154 = lean_box(0); +return x_154; +} +else +{ +lean_object* x_155; lean_object* x_156; uint8_t x_157; +x_155 = lean_ctor_get(x_149, 0); +lean_inc(x_155); +lean_dec(x_149); +x_156 = lean_ctor_get(x_151, 0); +lean_inc(x_156); +lean_dec(x_151); +x_157 = !lean_is_exclusive(x_153); +if (x_157 == 0) +{ +lean_object* x_158; lean_object* x_159; +x_158 = lean_ctor_get(x_153, 0); +x_159 = l_Lean_Name_mkStr3(x_155, x_156, x_158); +lean_ctor_set(x_153, 0, x_159); +return x_153; +} +else +{ +lean_object* x_160; lean_object* x_161; lean_object* x_162; +x_160 = lean_ctor_get(x_153, 0); +lean_inc(x_160); +lean_dec(x_153); +x_161 = l_Lean_Name_mkStr3(x_155, x_156, x_160); +x_162 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_162, 0, x_161); +return x_162; +} +} +} +else +{ +lean_object* x_163; +lean_dec(x_151); +lean_dec(x_149); +lean_dec(x_134); +x_163 = lean_box(0); +return x_163; +} +} +} +else +{ +lean_object* x_164; +lean_dec(x_149); +lean_dec(x_135); +lean_dec(x_134); +x_164 = lean_box(0); +return x_164; +} +} +} +else +{ +lean_object* x_165; +lean_dec(x_136); +lean_dec(x_135); +lean_dec(x_134); +x_165 = lean_box(0); +return x_165; +} +} +} +} +} +else +{ +lean_object* x_166; +lean_dec(x_133); +lean_dec(x_132); +lean_dec(x_131); +lean_dec(x_130); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_166 = lean_box(0); +return x_166; +} +} +else +{ +lean_object* x_167; +lean_dec(x_132); +lean_dec(x_131); +lean_dec(x_130); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_167 = lean_box(0); +return x_167; +} +} +else +{ +lean_object* x_168; +lean_dec(x_131); +lean_dec(x_130); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_168 = lean_box(0); +return x_168; +} +} +else +{ +lean_object* x_169; +lean_dec(x_130); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_169 = lean_box(0); +return x_169; +} +} +case 5: +{ +lean_object* x_170; +x_170 = lean_ctor_get(x_129, 0); +lean_inc(x_170); +switch (lean_obj_tag(x_170)) { +case 4: +{ +lean_object* x_171; +x_171 = lean_ctor_get(x_170, 0); +lean_inc(x_171); +lean_dec(x_170); +if (lean_obj_tag(x_171) == 1) +{ +lean_object* x_172; +x_172 = lean_ctor_get(x_171, 0); +lean_inc(x_172); +if (lean_obj_tag(x_172) == 1) +{ +lean_object* x_173; +x_173 = lean_ctor_get(x_172, 0); +lean_inc(x_173); +if (lean_obj_tag(x_173) == 1) +{ +lean_object* x_174; +x_174 = lean_ctor_get(x_173, 0); +lean_inc(x_174); +if (lean_obj_tag(x_174) == 0) +{ +lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; uint8_t x_183; +x_175 = lean_ctor_get(x_1, 1); +lean_inc(x_175); +lean_dec(x_1); +x_176 = lean_ctor_get(x_23, 1); +lean_inc(x_176); +lean_dec(x_23); +x_177 = lean_ctor_get(x_56, 1); +lean_inc(x_177); +lean_dec(x_56); +x_178 = lean_ctor_get(x_129, 1); +lean_inc(x_178); +lean_dec(x_129); +x_179 = lean_ctor_get(x_171, 1); +lean_inc(x_179); +lean_dec(x_171); +x_180 = lean_ctor_get(x_172, 1); +lean_inc(x_180); +lean_dec(x_172); +x_181 = lean_ctor_get(x_173, 1); +lean_inc(x_181); +lean_dec(x_173); +x_182 = l_Lean_Expr_name_x3f___closed__1; +x_183 = lean_string_dec_eq(x_181, x_182); +lean_dec(x_181); +if (x_183 == 0) +{ +lean_object* x_184; +lean_dec(x_180); +lean_dec(x_179); +lean_dec(x_178); +lean_dec(x_177); +lean_dec(x_176); +lean_dec(x_175); +x_184 = lean_box(0); +return x_184; +} +else +{ +lean_object* x_185; uint8_t x_186; +x_185 = l_Lean_Expr_name_x3f___closed__2; +x_186 = lean_string_dec_eq(x_180, x_185); +lean_dec(x_180); +if (x_186 == 0) +{ +lean_object* x_187; +lean_dec(x_179); +lean_dec(x_178); +lean_dec(x_177); +lean_dec(x_176); +lean_dec(x_175); +x_187 = lean_box(0); +return x_187; +} +else +{ +lean_object* x_188; uint8_t x_189; +x_188 = l_Lean_Expr_name_x3f___closed__10; +x_189 = lean_string_dec_eq(x_179, x_188); +lean_dec(x_179); +if (x_189 == 0) +{ +lean_object* x_190; +lean_dec(x_178); +lean_dec(x_177); +lean_dec(x_176); +lean_dec(x_175); +x_190 = lean_box(0); +return x_190; +} +else +{ +if (lean_obj_tag(x_178) == 9) +{ +lean_object* x_191; +x_191 = lean_ctor_get(x_178, 0); +lean_inc(x_191); +lean_dec(x_178); +if (lean_obj_tag(x_191) == 0) +{ +lean_object* x_192; +lean_dec(x_191); +lean_dec(x_177); +lean_dec(x_176); +lean_dec(x_175); +x_192 = lean_box(0); +return x_192; +} +else +{ +if (lean_obj_tag(x_177) == 9) +{ +lean_object* x_193; +x_193 = lean_ctor_get(x_177, 0); +lean_inc(x_193); +lean_dec(x_177); +if (lean_obj_tag(x_193) == 0) +{ +lean_object* x_194; +lean_dec(x_193); +lean_dec(x_191); +lean_dec(x_176); +lean_dec(x_175); +x_194 = lean_box(0); +return x_194; +} +else +{ +if (lean_obj_tag(x_176) == 9) +{ +lean_object* x_195; +x_195 = lean_ctor_get(x_176, 0); +lean_inc(x_195); +lean_dec(x_176); +if (lean_obj_tag(x_195) == 0) +{ +lean_object* x_196; +lean_dec(x_195); +lean_dec(x_193); +lean_dec(x_191); +lean_dec(x_175); +x_196 = lean_box(0); +return x_196; +} +else +{ +if (lean_obj_tag(x_175) == 9) +{ +lean_object* x_197; +x_197 = lean_ctor_get(x_175, 0); +lean_inc(x_197); +lean_dec(x_175); +if (lean_obj_tag(x_197) == 0) +{ +lean_object* x_198; +lean_dec(x_197); +lean_dec(x_195); +lean_dec(x_193); +lean_dec(x_191); +x_198 = lean_box(0); +return x_198; +} +else +{ +lean_object* x_199; lean_object* x_200; lean_object* x_201; uint8_t x_202; +x_199 = lean_ctor_get(x_191, 0); +lean_inc(x_199); +lean_dec(x_191); +x_200 = lean_ctor_get(x_193, 0); +lean_inc(x_200); +lean_dec(x_193); +x_201 = lean_ctor_get(x_195, 0); +lean_inc(x_201); +lean_dec(x_195); +x_202 = !lean_is_exclusive(x_197); +if (x_202 == 0) +{ +lean_object* x_203; lean_object* x_204; +x_203 = lean_ctor_get(x_197, 0); +x_204 = l_Lean_Name_mkStr4(x_199, x_200, x_201, x_203); +lean_ctor_set(x_197, 0, x_204); +return x_197; +} +else +{ +lean_object* x_205; lean_object* x_206; lean_object* x_207; +x_205 = lean_ctor_get(x_197, 0); +lean_inc(x_205); +lean_dec(x_197); +x_206 = l_Lean_Name_mkStr4(x_199, x_200, x_201, x_205); +x_207 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_207, 0, x_206); +return x_207; +} +} +} +else +{ +lean_object* x_208; +lean_dec(x_195); +lean_dec(x_193); +lean_dec(x_191); +lean_dec(x_175); +x_208 = lean_box(0); +return x_208; +} +} +} +else +{ +lean_object* x_209; +lean_dec(x_193); +lean_dec(x_191); +lean_dec(x_176); +lean_dec(x_175); +x_209 = lean_box(0); +return x_209; +} +} +} +else +{ +lean_object* x_210; +lean_dec(x_191); +lean_dec(x_177); +lean_dec(x_176); +lean_dec(x_175); +x_210 = lean_box(0); +return x_210; +} +} +} +else +{ +lean_object* x_211; +lean_dec(x_178); +lean_dec(x_177); +lean_dec(x_176); +lean_dec(x_175); +x_211 = lean_box(0); +return x_211; +} +} +} +} +} +else +{ +lean_object* x_212; +lean_dec(x_174); +lean_dec(x_173); +lean_dec(x_172); +lean_dec(x_171); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_212 = lean_box(0); +return x_212; +} +} +else +{ +lean_object* x_213; +lean_dec(x_173); +lean_dec(x_172); +lean_dec(x_171); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_213 = lean_box(0); +return x_213; +} +} +else +{ +lean_object* x_214; +lean_dec(x_172); +lean_dec(x_171); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_214 = lean_box(0); +return x_214; +} +} +else +{ +lean_object* x_215; +lean_dec(x_171); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_215 = lean_box(0); +return x_215; +} +} +case 5: +{ +lean_object* x_216; +x_216 = lean_ctor_get(x_170, 0); +lean_inc(x_216); +switch (lean_obj_tag(x_216)) { +case 4: +{ +lean_object* x_217; +x_217 = lean_ctor_get(x_216, 0); +lean_inc(x_217); +lean_dec(x_216); +if (lean_obj_tag(x_217) == 1) +{ +lean_object* x_218; +x_218 = lean_ctor_get(x_217, 0); +lean_inc(x_218); +if (lean_obj_tag(x_218) == 1) +{ +lean_object* x_219; +x_219 = lean_ctor_get(x_218, 0); +lean_inc(x_219); +if (lean_obj_tag(x_219) == 1) +{ +lean_object* x_220; +x_220 = lean_ctor_get(x_219, 0); +lean_inc(x_220); +if (lean_obj_tag(x_220) == 0) +{ +lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; uint8_t x_230; +x_221 = lean_ctor_get(x_1, 1); +lean_inc(x_221); +lean_dec(x_1); +x_222 = lean_ctor_get(x_23, 1); +lean_inc(x_222); +lean_dec(x_23); +x_223 = lean_ctor_get(x_56, 1); +lean_inc(x_223); +lean_dec(x_56); +x_224 = lean_ctor_get(x_129, 1); +lean_inc(x_224); +lean_dec(x_129); +x_225 = lean_ctor_get(x_170, 1); +lean_inc(x_225); +lean_dec(x_170); +x_226 = lean_ctor_get(x_217, 1); +lean_inc(x_226); +lean_dec(x_217); +x_227 = lean_ctor_get(x_218, 1); +lean_inc(x_227); +lean_dec(x_218); +x_228 = lean_ctor_get(x_219, 1); +lean_inc(x_228); +lean_dec(x_219); +x_229 = l_Lean_Expr_name_x3f___closed__1; +x_230 = lean_string_dec_eq(x_228, x_229); +lean_dec(x_228); +if (x_230 == 0) +{ +lean_object* x_231; +lean_dec(x_227); +lean_dec(x_226); +lean_dec(x_225); +lean_dec(x_224); +lean_dec(x_223); +lean_dec(x_222); +lean_dec(x_221); +x_231 = lean_box(0); +return x_231; +} +else +{ +lean_object* x_232; uint8_t x_233; +x_232 = l_Lean_Expr_name_x3f___closed__2; +x_233 = lean_string_dec_eq(x_227, x_232); +lean_dec(x_227); +if (x_233 == 0) +{ +lean_object* x_234; +lean_dec(x_226); +lean_dec(x_225); +lean_dec(x_224); +lean_dec(x_223); +lean_dec(x_222); +lean_dec(x_221); +x_234 = lean_box(0); +return x_234; +} +else +{ +lean_object* x_235; uint8_t x_236; +x_235 = l_Lean_Expr_name_x3f___closed__11; +x_236 = lean_string_dec_eq(x_226, x_235); +lean_dec(x_226); +if (x_236 == 0) +{ +lean_object* x_237; +lean_dec(x_225); +lean_dec(x_224); +lean_dec(x_223); +lean_dec(x_222); +lean_dec(x_221); +x_237 = lean_box(0); +return x_237; +} +else +{ +if (lean_obj_tag(x_225) == 9) +{ +lean_object* x_238; +x_238 = lean_ctor_get(x_225, 0); +lean_inc(x_238); +lean_dec(x_225); +if (lean_obj_tag(x_238) == 0) +{ +lean_object* x_239; +lean_dec(x_238); +lean_dec(x_224); +lean_dec(x_223); +lean_dec(x_222); +lean_dec(x_221); +x_239 = lean_box(0); +return x_239; +} +else +{ +if (lean_obj_tag(x_224) == 9) +{ +lean_object* x_240; +x_240 = lean_ctor_get(x_224, 0); +lean_inc(x_240); +lean_dec(x_224); +if (lean_obj_tag(x_240) == 0) +{ +lean_object* x_241; +lean_dec(x_240); +lean_dec(x_238); +lean_dec(x_223); +lean_dec(x_222); +lean_dec(x_221); +x_241 = lean_box(0); +return x_241; +} +else +{ +if (lean_obj_tag(x_223) == 9) +{ +lean_object* x_242; +x_242 = lean_ctor_get(x_223, 0); +lean_inc(x_242); +lean_dec(x_223); +if (lean_obj_tag(x_242) == 0) +{ +lean_object* x_243; +lean_dec(x_242); +lean_dec(x_240); +lean_dec(x_238); +lean_dec(x_222); +lean_dec(x_221); +x_243 = lean_box(0); +return x_243; +} +else +{ +if (lean_obj_tag(x_222) == 9) +{ +lean_object* x_244; +x_244 = lean_ctor_get(x_222, 0); +lean_inc(x_244); +lean_dec(x_222); +if (lean_obj_tag(x_244) == 0) +{ +lean_object* x_245; +lean_dec(x_244); +lean_dec(x_242); +lean_dec(x_240); +lean_dec(x_238); +lean_dec(x_221); +x_245 = lean_box(0); +return x_245; +} +else +{ +if (lean_obj_tag(x_221) == 9) +{ +lean_object* x_246; +x_246 = lean_ctor_get(x_221, 0); +lean_inc(x_246); +lean_dec(x_221); +if (lean_obj_tag(x_246) == 0) +{ +lean_object* x_247; +lean_dec(x_246); +lean_dec(x_244); +lean_dec(x_242); +lean_dec(x_240); +lean_dec(x_238); +x_247 = lean_box(0); +return x_247; +} +else +{ +lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; uint8_t x_252; +x_248 = lean_ctor_get(x_238, 0); +lean_inc(x_248); +lean_dec(x_238); +x_249 = lean_ctor_get(x_240, 0); +lean_inc(x_249); +lean_dec(x_240); +x_250 = lean_ctor_get(x_242, 0); +lean_inc(x_250); +lean_dec(x_242); +x_251 = lean_ctor_get(x_244, 0); +lean_inc(x_251); +lean_dec(x_244); +x_252 = !lean_is_exclusive(x_246); +if (x_252 == 0) +{ +lean_object* x_253; lean_object* x_254; +x_253 = lean_ctor_get(x_246, 0); +x_254 = l_Lean_Name_mkStr5(x_248, x_249, x_250, x_251, x_253); +lean_ctor_set(x_246, 0, x_254); +return x_246; +} +else +{ +lean_object* x_255; lean_object* x_256; lean_object* x_257; +x_255 = lean_ctor_get(x_246, 0); +lean_inc(x_255); +lean_dec(x_246); +x_256 = l_Lean_Name_mkStr5(x_248, x_249, x_250, x_251, x_255); +x_257 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_257, 0, x_256); +return x_257; +} +} +} +else +{ +lean_object* x_258; +lean_dec(x_244); +lean_dec(x_242); +lean_dec(x_240); +lean_dec(x_238); +lean_dec(x_221); +x_258 = lean_box(0); +return x_258; +} +} +} +else +{ +lean_object* x_259; +lean_dec(x_242); +lean_dec(x_240); +lean_dec(x_238); +lean_dec(x_222); +lean_dec(x_221); +x_259 = lean_box(0); +return x_259; +} +} +} +else +{ +lean_object* x_260; +lean_dec(x_240); +lean_dec(x_238); +lean_dec(x_223); +lean_dec(x_222); +lean_dec(x_221); +x_260 = lean_box(0); +return x_260; +} +} +} +else +{ +lean_object* x_261; +lean_dec(x_238); +lean_dec(x_224); +lean_dec(x_223); +lean_dec(x_222); +lean_dec(x_221); +x_261 = lean_box(0); +return x_261; +} +} +} +else +{ +lean_object* x_262; +lean_dec(x_225); +lean_dec(x_224); +lean_dec(x_223); +lean_dec(x_222); +lean_dec(x_221); +x_262 = lean_box(0); +return x_262; +} +} +} +} +} +else +{ +lean_object* x_263; +lean_dec(x_220); +lean_dec(x_219); +lean_dec(x_218); +lean_dec(x_217); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_263 = lean_box(0); +return x_263; +} +} +else +{ +lean_object* x_264; +lean_dec(x_219); +lean_dec(x_218); +lean_dec(x_217); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_264 = lean_box(0); +return x_264; +} +} +else +{ +lean_object* x_265; +lean_dec(x_218); +lean_dec(x_217); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_265 = lean_box(0); +return x_265; +} +} +else +{ +lean_object* x_266; +lean_dec(x_217); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_266 = lean_box(0); +return x_266; +} +} +case 5: +{ +lean_object* x_267; +x_267 = lean_ctor_get(x_216, 0); +lean_inc(x_267); +switch (lean_obj_tag(x_267)) { +case 4: +{ +lean_object* x_268; +x_268 = lean_ctor_get(x_267, 0); +lean_inc(x_268); +lean_dec(x_267); +if (lean_obj_tag(x_268) == 1) +{ +lean_object* x_269; +x_269 = lean_ctor_get(x_268, 0); +lean_inc(x_269); +if (lean_obj_tag(x_269) == 1) +{ +lean_object* x_270; +x_270 = lean_ctor_get(x_269, 0); +lean_inc(x_270); +if (lean_obj_tag(x_270) == 1) +{ +lean_object* x_271; +x_271 = lean_ctor_get(x_270, 0); +lean_inc(x_271); +if (lean_obj_tag(x_271) == 0) +{ +lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; uint8_t x_282; +x_272 = lean_ctor_get(x_1, 1); +lean_inc(x_272); +lean_dec(x_1); +x_273 = lean_ctor_get(x_23, 1); +lean_inc(x_273); +lean_dec(x_23); +x_274 = lean_ctor_get(x_56, 1); +lean_inc(x_274); +lean_dec(x_56); +x_275 = lean_ctor_get(x_129, 1); +lean_inc(x_275); +lean_dec(x_129); +x_276 = lean_ctor_get(x_170, 1); +lean_inc(x_276); +lean_dec(x_170); +x_277 = lean_ctor_get(x_216, 1); +lean_inc(x_277); +lean_dec(x_216); +x_278 = lean_ctor_get(x_268, 1); +lean_inc(x_278); +lean_dec(x_268); +x_279 = lean_ctor_get(x_269, 1); +lean_inc(x_279); +lean_dec(x_269); +x_280 = lean_ctor_get(x_270, 1); +lean_inc(x_280); +lean_dec(x_270); +x_281 = l_Lean_Expr_name_x3f___closed__1; +x_282 = lean_string_dec_eq(x_280, x_281); +lean_dec(x_280); +if (x_282 == 0) +{ +lean_object* x_283; +lean_dec(x_279); +lean_dec(x_278); +lean_dec(x_277); +lean_dec(x_276); +lean_dec(x_275); +lean_dec(x_274); +lean_dec(x_273); +lean_dec(x_272); +x_283 = lean_box(0); +return x_283; +} +else +{ +lean_object* x_284; uint8_t x_285; +x_284 = l_Lean_Expr_name_x3f___closed__2; +x_285 = lean_string_dec_eq(x_279, x_284); +lean_dec(x_279); +if (x_285 == 0) +{ +lean_object* x_286; +lean_dec(x_278); +lean_dec(x_277); +lean_dec(x_276); +lean_dec(x_275); +lean_dec(x_274); +lean_dec(x_273); +lean_dec(x_272); +x_286 = lean_box(0); +return x_286; +} +else +{ +lean_object* x_287; uint8_t x_288; +x_287 = l_Lean_Expr_name_x3f___closed__12; +x_288 = lean_string_dec_eq(x_278, x_287); +lean_dec(x_278); +if (x_288 == 0) +{ +lean_object* x_289; +lean_dec(x_277); +lean_dec(x_276); +lean_dec(x_275); +lean_dec(x_274); +lean_dec(x_273); +lean_dec(x_272); +x_289 = lean_box(0); +return x_289; +} +else +{ +if (lean_obj_tag(x_277) == 9) +{ +lean_object* x_290; +x_290 = lean_ctor_get(x_277, 0); +lean_inc(x_290); +lean_dec(x_277); +if (lean_obj_tag(x_290) == 0) +{ +lean_object* x_291; +lean_dec(x_290); +lean_dec(x_276); +lean_dec(x_275); +lean_dec(x_274); +lean_dec(x_273); +lean_dec(x_272); +x_291 = lean_box(0); +return x_291; +} +else +{ +if (lean_obj_tag(x_276) == 9) +{ +lean_object* x_292; +x_292 = lean_ctor_get(x_276, 0); +lean_inc(x_292); +lean_dec(x_276); +if (lean_obj_tag(x_292) == 0) +{ +lean_object* x_293; +lean_dec(x_292); +lean_dec(x_290); +lean_dec(x_275); +lean_dec(x_274); +lean_dec(x_273); +lean_dec(x_272); +x_293 = lean_box(0); +return x_293; +} +else +{ +if (lean_obj_tag(x_275) == 9) +{ +lean_object* x_294; +x_294 = lean_ctor_get(x_275, 0); +lean_inc(x_294); +lean_dec(x_275); +if (lean_obj_tag(x_294) == 0) +{ +lean_object* x_295; +lean_dec(x_294); +lean_dec(x_292); +lean_dec(x_290); +lean_dec(x_274); +lean_dec(x_273); +lean_dec(x_272); +x_295 = lean_box(0); +return x_295; +} +else +{ +if (lean_obj_tag(x_274) == 9) +{ +lean_object* x_296; +x_296 = lean_ctor_get(x_274, 0); +lean_inc(x_296); +lean_dec(x_274); +if (lean_obj_tag(x_296) == 0) +{ +lean_object* x_297; +lean_dec(x_296); +lean_dec(x_294); +lean_dec(x_292); +lean_dec(x_290); +lean_dec(x_273); +lean_dec(x_272); +x_297 = lean_box(0); +return x_297; +} +else +{ +if (lean_obj_tag(x_273) == 9) +{ +lean_object* x_298; +x_298 = lean_ctor_get(x_273, 0); +lean_inc(x_298); +lean_dec(x_273); +if (lean_obj_tag(x_298) == 0) +{ +lean_object* x_299; +lean_dec(x_298); +lean_dec(x_296); +lean_dec(x_294); +lean_dec(x_292); +lean_dec(x_290); +lean_dec(x_272); +x_299 = lean_box(0); +return x_299; +} +else +{ +if (lean_obj_tag(x_272) == 9) +{ +lean_object* x_300; +x_300 = lean_ctor_get(x_272, 0); +lean_inc(x_300); +lean_dec(x_272); +if (lean_obj_tag(x_300) == 0) +{ +lean_object* x_301; +lean_dec(x_300); +lean_dec(x_298); +lean_dec(x_296); +lean_dec(x_294); +lean_dec(x_292); +lean_dec(x_290); +x_301 = lean_box(0); +return x_301; +} +else +{ +lean_object* x_302; lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; uint8_t x_307; +x_302 = lean_ctor_get(x_290, 0); +lean_inc(x_302); +lean_dec(x_290); +x_303 = lean_ctor_get(x_292, 0); +lean_inc(x_303); +lean_dec(x_292); +x_304 = lean_ctor_get(x_294, 0); +lean_inc(x_304); +lean_dec(x_294); +x_305 = lean_ctor_get(x_296, 0); +lean_inc(x_305); +lean_dec(x_296); +x_306 = lean_ctor_get(x_298, 0); +lean_inc(x_306); +lean_dec(x_298); +x_307 = !lean_is_exclusive(x_300); +if (x_307 == 0) +{ +lean_object* x_308; lean_object* x_309; +x_308 = lean_ctor_get(x_300, 0); +x_309 = l_Lean_Name_mkStr6(x_302, x_303, x_304, x_305, x_306, x_308); +lean_ctor_set(x_300, 0, x_309); +return x_300; +} +else +{ +lean_object* x_310; lean_object* x_311; lean_object* x_312; +x_310 = lean_ctor_get(x_300, 0); +lean_inc(x_310); +lean_dec(x_300); +x_311 = l_Lean_Name_mkStr6(x_302, x_303, x_304, x_305, x_306, x_310); +x_312 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_312, 0, x_311); +return x_312; +} +} +} +else +{ +lean_object* x_313; +lean_dec(x_298); +lean_dec(x_296); +lean_dec(x_294); +lean_dec(x_292); +lean_dec(x_290); +lean_dec(x_272); +x_313 = lean_box(0); +return x_313; +} +} +} +else +{ +lean_object* x_314; +lean_dec(x_296); +lean_dec(x_294); +lean_dec(x_292); +lean_dec(x_290); +lean_dec(x_273); +lean_dec(x_272); +x_314 = lean_box(0); +return x_314; +} +} +} +else +{ +lean_object* x_315; +lean_dec(x_294); +lean_dec(x_292); +lean_dec(x_290); +lean_dec(x_274); +lean_dec(x_273); +lean_dec(x_272); +x_315 = lean_box(0); +return x_315; +} +} +} +else +{ +lean_object* x_316; +lean_dec(x_292); +lean_dec(x_290); +lean_dec(x_275); +lean_dec(x_274); +lean_dec(x_273); +lean_dec(x_272); +x_316 = lean_box(0); +return x_316; +} +} +} +else +{ +lean_object* x_317; +lean_dec(x_290); +lean_dec(x_276); +lean_dec(x_275); +lean_dec(x_274); +lean_dec(x_273); +lean_dec(x_272); +x_317 = lean_box(0); +return x_317; +} +} +} +else +{ +lean_object* x_318; +lean_dec(x_277); +lean_dec(x_276); +lean_dec(x_275); +lean_dec(x_274); +lean_dec(x_273); +lean_dec(x_272); +x_318 = lean_box(0); +return x_318; +} +} +} +} +} +else +{ +lean_object* x_319; +lean_dec(x_271); +lean_dec(x_270); +lean_dec(x_269); +lean_dec(x_268); +lean_dec(x_216); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_319 = lean_box(0); +return x_319; +} +} +else +{ +lean_object* x_320; +lean_dec(x_270); +lean_dec(x_269); +lean_dec(x_268); +lean_dec(x_216); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_320 = lean_box(0); +return x_320; +} +} +else +{ +lean_object* x_321; +lean_dec(x_269); +lean_dec(x_268); +lean_dec(x_216); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_321 = lean_box(0); +return x_321; +} +} +else +{ +lean_object* x_322; +lean_dec(x_268); +lean_dec(x_216); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_322 = lean_box(0); +return x_322; +} +} +case 5: +{ +lean_object* x_323; +x_323 = lean_ctor_get(x_267, 0); +lean_inc(x_323); +switch (lean_obj_tag(x_323)) { +case 4: +{ +lean_object* x_324; +x_324 = lean_ctor_get(x_323, 0); +lean_inc(x_324); +lean_dec(x_323); +if (lean_obj_tag(x_324) == 1) +{ +lean_object* x_325; +x_325 = lean_ctor_get(x_324, 0); +lean_inc(x_325); +if (lean_obj_tag(x_325) == 1) +{ +lean_object* x_326; +x_326 = lean_ctor_get(x_325, 0); +lean_inc(x_326); +if (lean_obj_tag(x_326) == 1) +{ +lean_object* x_327; +x_327 = lean_ctor_get(x_326, 0); +lean_inc(x_327); +if (lean_obj_tag(x_327) == 0) +{ +lean_object* x_328; lean_object* x_329; lean_object* x_330; lean_object* x_331; lean_object* x_332; lean_object* x_333; lean_object* x_334; lean_object* x_335; lean_object* x_336; lean_object* x_337; lean_object* x_338; uint8_t x_339; +x_328 = lean_ctor_get(x_1, 1); +lean_inc(x_328); +lean_dec(x_1); +x_329 = lean_ctor_get(x_23, 1); +lean_inc(x_329); +lean_dec(x_23); +x_330 = lean_ctor_get(x_56, 1); +lean_inc(x_330); +lean_dec(x_56); +x_331 = lean_ctor_get(x_129, 1); +lean_inc(x_331); +lean_dec(x_129); +x_332 = lean_ctor_get(x_170, 1); +lean_inc(x_332); +lean_dec(x_170); +x_333 = lean_ctor_get(x_216, 1); +lean_inc(x_333); +lean_dec(x_216); +x_334 = lean_ctor_get(x_267, 1); +lean_inc(x_334); +lean_dec(x_267); +x_335 = lean_ctor_get(x_324, 1); +lean_inc(x_335); +lean_dec(x_324); +x_336 = lean_ctor_get(x_325, 1); +lean_inc(x_336); +lean_dec(x_325); +x_337 = lean_ctor_get(x_326, 1); +lean_inc(x_337); +lean_dec(x_326); +x_338 = l_Lean_Expr_name_x3f___closed__1; +x_339 = lean_string_dec_eq(x_337, x_338); +lean_dec(x_337); +if (x_339 == 0) +{ +lean_object* x_340; +lean_dec(x_336); +lean_dec(x_335); +lean_dec(x_334); +lean_dec(x_333); +lean_dec(x_332); +lean_dec(x_331); +lean_dec(x_330); +lean_dec(x_329); +lean_dec(x_328); +x_340 = lean_box(0); +return x_340; +} +else +{ +lean_object* x_341; uint8_t x_342; +x_341 = l_Lean_Expr_name_x3f___closed__2; +x_342 = lean_string_dec_eq(x_336, x_341); +lean_dec(x_336); +if (x_342 == 0) +{ +lean_object* x_343; +lean_dec(x_335); +lean_dec(x_334); +lean_dec(x_333); +lean_dec(x_332); +lean_dec(x_331); +lean_dec(x_330); +lean_dec(x_329); +lean_dec(x_328); +x_343 = lean_box(0); +return x_343; +} +else +{ +lean_object* x_344; uint8_t x_345; +x_344 = l_Lean_Expr_name_x3f___closed__13; +x_345 = lean_string_dec_eq(x_335, x_344); +lean_dec(x_335); +if (x_345 == 0) +{ +lean_object* x_346; +lean_dec(x_334); +lean_dec(x_333); +lean_dec(x_332); +lean_dec(x_331); +lean_dec(x_330); +lean_dec(x_329); +lean_dec(x_328); +x_346 = lean_box(0); +return x_346; +} +else +{ +if (lean_obj_tag(x_334) == 9) +{ +lean_object* x_347; +x_347 = lean_ctor_get(x_334, 0); +lean_inc(x_347); +lean_dec(x_334); +if (lean_obj_tag(x_347) == 0) +{ +lean_object* x_348; +lean_dec(x_347); +lean_dec(x_333); +lean_dec(x_332); +lean_dec(x_331); +lean_dec(x_330); +lean_dec(x_329); +lean_dec(x_328); +x_348 = lean_box(0); +return x_348; +} +else +{ +if (lean_obj_tag(x_333) == 9) +{ +lean_object* x_349; +x_349 = lean_ctor_get(x_333, 0); +lean_inc(x_349); +lean_dec(x_333); +if (lean_obj_tag(x_349) == 0) +{ +lean_object* x_350; +lean_dec(x_349); +lean_dec(x_347); +lean_dec(x_332); +lean_dec(x_331); +lean_dec(x_330); +lean_dec(x_329); +lean_dec(x_328); +x_350 = lean_box(0); +return x_350; +} +else +{ +if (lean_obj_tag(x_332) == 9) +{ +lean_object* x_351; +x_351 = lean_ctor_get(x_332, 0); +lean_inc(x_351); +lean_dec(x_332); +if (lean_obj_tag(x_351) == 0) +{ +lean_object* x_352; +lean_dec(x_351); +lean_dec(x_349); +lean_dec(x_347); +lean_dec(x_331); +lean_dec(x_330); +lean_dec(x_329); +lean_dec(x_328); +x_352 = lean_box(0); +return x_352; +} +else +{ +if (lean_obj_tag(x_331) == 9) +{ +lean_object* x_353; +x_353 = lean_ctor_get(x_331, 0); +lean_inc(x_353); +lean_dec(x_331); +if (lean_obj_tag(x_353) == 0) +{ +lean_object* x_354; +lean_dec(x_353); +lean_dec(x_351); +lean_dec(x_349); +lean_dec(x_347); +lean_dec(x_330); +lean_dec(x_329); +lean_dec(x_328); +x_354 = lean_box(0); +return x_354; +} +else +{ +if (lean_obj_tag(x_330) == 9) +{ +lean_object* x_355; +x_355 = lean_ctor_get(x_330, 0); +lean_inc(x_355); +lean_dec(x_330); +if (lean_obj_tag(x_355) == 0) +{ +lean_object* x_356; +lean_dec(x_355); +lean_dec(x_353); +lean_dec(x_351); +lean_dec(x_349); +lean_dec(x_347); +lean_dec(x_329); +lean_dec(x_328); +x_356 = lean_box(0); +return x_356; +} +else +{ +if (lean_obj_tag(x_329) == 9) +{ +lean_object* x_357; +x_357 = lean_ctor_get(x_329, 0); +lean_inc(x_357); +lean_dec(x_329); +if (lean_obj_tag(x_357) == 0) +{ +lean_object* x_358; +lean_dec(x_357); +lean_dec(x_355); +lean_dec(x_353); +lean_dec(x_351); +lean_dec(x_349); +lean_dec(x_347); +lean_dec(x_328); +x_358 = lean_box(0); +return x_358; +} +else +{ +if (lean_obj_tag(x_328) == 9) +{ +lean_object* x_359; +x_359 = lean_ctor_get(x_328, 0); +lean_inc(x_359); +lean_dec(x_328); +if (lean_obj_tag(x_359) == 0) +{ +lean_object* x_360; +lean_dec(x_359); +lean_dec(x_357); +lean_dec(x_355); +lean_dec(x_353); +lean_dec(x_351); +lean_dec(x_349); +lean_dec(x_347); +x_360 = lean_box(0); +return x_360; +} +else +{ +lean_object* x_361; lean_object* x_362; lean_object* x_363; lean_object* x_364; lean_object* x_365; lean_object* x_366; uint8_t x_367; +x_361 = lean_ctor_get(x_347, 0); +lean_inc(x_361); +lean_dec(x_347); +x_362 = lean_ctor_get(x_349, 0); +lean_inc(x_362); +lean_dec(x_349); +x_363 = lean_ctor_get(x_351, 0); +lean_inc(x_363); +lean_dec(x_351); +x_364 = lean_ctor_get(x_353, 0); +lean_inc(x_364); +lean_dec(x_353); +x_365 = lean_ctor_get(x_355, 0); +lean_inc(x_365); +lean_dec(x_355); +x_366 = lean_ctor_get(x_357, 0); +lean_inc(x_366); +lean_dec(x_357); +x_367 = !lean_is_exclusive(x_359); +if (x_367 == 0) +{ +lean_object* x_368; lean_object* x_369; +x_368 = lean_ctor_get(x_359, 0); +x_369 = l_Lean_Name_mkStr7(x_361, x_362, x_363, x_364, x_365, x_366, x_368); +lean_ctor_set(x_359, 0, x_369); +return x_359; +} +else +{ +lean_object* x_370; lean_object* x_371; lean_object* x_372; +x_370 = lean_ctor_get(x_359, 0); +lean_inc(x_370); +lean_dec(x_359); +x_371 = l_Lean_Name_mkStr7(x_361, x_362, x_363, x_364, x_365, x_366, x_370); +x_372 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_372, 0, x_371); +return x_372; +} +} +} +else +{ +lean_object* x_373; +lean_dec(x_357); +lean_dec(x_355); +lean_dec(x_353); +lean_dec(x_351); +lean_dec(x_349); +lean_dec(x_347); +lean_dec(x_328); +x_373 = lean_box(0); +return x_373; +} +} +} +else +{ +lean_object* x_374; +lean_dec(x_355); +lean_dec(x_353); +lean_dec(x_351); +lean_dec(x_349); +lean_dec(x_347); +lean_dec(x_329); +lean_dec(x_328); +x_374 = lean_box(0); +return x_374; +} +} +} +else +{ +lean_object* x_375; +lean_dec(x_353); +lean_dec(x_351); +lean_dec(x_349); +lean_dec(x_347); +lean_dec(x_330); +lean_dec(x_329); +lean_dec(x_328); +x_375 = lean_box(0); +return x_375; +} +} +} +else +{ +lean_object* x_376; +lean_dec(x_351); +lean_dec(x_349); +lean_dec(x_347); +lean_dec(x_331); +lean_dec(x_330); +lean_dec(x_329); +lean_dec(x_328); +x_376 = lean_box(0); +return x_376; +} +} +} +else +{ +lean_object* x_377; +lean_dec(x_349); +lean_dec(x_347); +lean_dec(x_332); +lean_dec(x_331); +lean_dec(x_330); +lean_dec(x_329); +lean_dec(x_328); +x_377 = lean_box(0); +return x_377; +} +} +} +else +{ +lean_object* x_378; +lean_dec(x_347); +lean_dec(x_333); +lean_dec(x_332); +lean_dec(x_331); +lean_dec(x_330); +lean_dec(x_329); +lean_dec(x_328); +x_378 = lean_box(0); +return x_378; +} +} +} +else +{ +lean_object* x_379; +lean_dec(x_334); +lean_dec(x_333); +lean_dec(x_332); +lean_dec(x_331); +lean_dec(x_330); +lean_dec(x_329); +lean_dec(x_328); +x_379 = lean_box(0); +return x_379; +} +} +} +} +} +else +{ +lean_object* x_380; +lean_dec(x_327); +lean_dec(x_326); +lean_dec(x_325); +lean_dec(x_324); +lean_dec(x_267); +lean_dec(x_216); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_380 = lean_box(0); +return x_380; +} +} +else +{ +lean_object* x_381; +lean_dec(x_326); +lean_dec(x_325); +lean_dec(x_324); +lean_dec(x_267); +lean_dec(x_216); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_381 = lean_box(0); +return x_381; +} +} +else +{ +lean_object* x_382; +lean_dec(x_325); +lean_dec(x_324); +lean_dec(x_267); +lean_dec(x_216); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_382 = lean_box(0); +return x_382; +} +} +else +{ +lean_object* x_383; +lean_dec(x_324); +lean_dec(x_267); +lean_dec(x_216); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_383 = lean_box(0); +return x_383; +} +} +case 5: +{ +lean_object* x_384; +x_384 = lean_ctor_get(x_323, 0); +lean_inc(x_384); +if (lean_obj_tag(x_384) == 4) +{ +lean_object* x_385; +x_385 = lean_ctor_get(x_384, 0); +lean_inc(x_385); +lean_dec(x_384); +if (lean_obj_tag(x_385) == 1) +{ +lean_object* x_386; +x_386 = lean_ctor_get(x_385, 0); +lean_inc(x_386); +if (lean_obj_tag(x_386) == 1) +{ +lean_object* x_387; +x_387 = lean_ctor_get(x_386, 0); +lean_inc(x_387); +if (lean_obj_tag(x_387) == 1) +{ +lean_object* x_388; +x_388 = lean_ctor_get(x_387, 0); +lean_inc(x_388); +if (lean_obj_tag(x_388) == 0) +{ +lean_object* x_389; lean_object* x_390; lean_object* x_391; lean_object* x_392; lean_object* x_393; lean_object* x_394; lean_object* x_395; lean_object* x_396; lean_object* x_397; lean_object* x_398; lean_object* x_399; lean_object* x_400; uint8_t x_401; +x_389 = lean_ctor_get(x_1, 1); +lean_inc(x_389); +lean_dec(x_1); +x_390 = lean_ctor_get(x_23, 1); +lean_inc(x_390); +lean_dec(x_23); +x_391 = lean_ctor_get(x_56, 1); +lean_inc(x_391); +lean_dec(x_56); +x_392 = lean_ctor_get(x_129, 1); +lean_inc(x_392); +lean_dec(x_129); +x_393 = lean_ctor_get(x_170, 1); +lean_inc(x_393); +lean_dec(x_170); +x_394 = lean_ctor_get(x_216, 1); +lean_inc(x_394); +lean_dec(x_216); +x_395 = lean_ctor_get(x_267, 1); +lean_inc(x_395); +lean_dec(x_267); +x_396 = lean_ctor_get(x_323, 1); +lean_inc(x_396); +lean_dec(x_323); +x_397 = lean_ctor_get(x_385, 1); +lean_inc(x_397); +lean_dec(x_385); +x_398 = lean_ctor_get(x_386, 1); +lean_inc(x_398); +lean_dec(x_386); +x_399 = lean_ctor_get(x_387, 1); +lean_inc(x_399); +lean_dec(x_387); +x_400 = l_Lean_Expr_name_x3f___closed__1; +x_401 = lean_string_dec_eq(x_399, x_400); +lean_dec(x_399); +if (x_401 == 0) +{ +lean_object* x_402; +lean_dec(x_398); +lean_dec(x_397); +lean_dec(x_396); +lean_dec(x_395); +lean_dec(x_394); +lean_dec(x_393); +lean_dec(x_392); +lean_dec(x_391); +lean_dec(x_390); +lean_dec(x_389); +x_402 = lean_box(0); +return x_402; +} +else +{ +lean_object* x_403; uint8_t x_404; +x_403 = l_Lean_Expr_name_x3f___closed__2; +x_404 = lean_string_dec_eq(x_398, x_403); +lean_dec(x_398); +if (x_404 == 0) +{ +lean_object* x_405; +lean_dec(x_397); +lean_dec(x_396); +lean_dec(x_395); +lean_dec(x_394); +lean_dec(x_393); +lean_dec(x_392); +lean_dec(x_391); +lean_dec(x_390); +lean_dec(x_389); +x_405 = lean_box(0); +return x_405; +} +else +{ +lean_object* x_406; uint8_t x_407; +x_406 = l_Lean_Expr_name_x3f___closed__14; +x_407 = lean_string_dec_eq(x_397, x_406); +lean_dec(x_397); +if (x_407 == 0) +{ +lean_object* x_408; +lean_dec(x_396); +lean_dec(x_395); +lean_dec(x_394); +lean_dec(x_393); +lean_dec(x_392); +lean_dec(x_391); +lean_dec(x_390); +lean_dec(x_389); +x_408 = lean_box(0); +return x_408; +} +else +{ +if (lean_obj_tag(x_396) == 9) +{ +lean_object* x_409; +x_409 = lean_ctor_get(x_396, 0); +lean_inc(x_409); +lean_dec(x_396); +if (lean_obj_tag(x_409) == 0) +{ +lean_object* x_410; +lean_dec(x_409); +lean_dec(x_395); +lean_dec(x_394); +lean_dec(x_393); +lean_dec(x_392); +lean_dec(x_391); +lean_dec(x_390); +lean_dec(x_389); +x_410 = lean_box(0); +return x_410; +} +else +{ +if (lean_obj_tag(x_395) == 9) +{ +lean_object* x_411; +x_411 = lean_ctor_get(x_395, 0); +lean_inc(x_411); +lean_dec(x_395); +if (lean_obj_tag(x_411) == 0) +{ +lean_object* x_412; +lean_dec(x_411); +lean_dec(x_409); +lean_dec(x_394); +lean_dec(x_393); +lean_dec(x_392); +lean_dec(x_391); +lean_dec(x_390); +lean_dec(x_389); +x_412 = lean_box(0); +return x_412; +} +else +{ +if (lean_obj_tag(x_394) == 9) +{ +lean_object* x_413; +x_413 = lean_ctor_get(x_394, 0); +lean_inc(x_413); +lean_dec(x_394); +if (lean_obj_tag(x_413) == 0) +{ +lean_object* x_414; +lean_dec(x_413); +lean_dec(x_411); +lean_dec(x_409); +lean_dec(x_393); +lean_dec(x_392); +lean_dec(x_391); +lean_dec(x_390); +lean_dec(x_389); +x_414 = lean_box(0); +return x_414; +} +else +{ +if (lean_obj_tag(x_393) == 9) +{ +lean_object* x_415; +x_415 = lean_ctor_get(x_393, 0); +lean_inc(x_415); +lean_dec(x_393); +if (lean_obj_tag(x_415) == 0) +{ +lean_object* x_416; +lean_dec(x_415); +lean_dec(x_413); +lean_dec(x_411); +lean_dec(x_409); +lean_dec(x_392); +lean_dec(x_391); +lean_dec(x_390); +lean_dec(x_389); +x_416 = lean_box(0); +return x_416; +} +else +{ +if (lean_obj_tag(x_392) == 9) +{ +lean_object* x_417; +x_417 = lean_ctor_get(x_392, 0); +lean_inc(x_417); +lean_dec(x_392); +if (lean_obj_tag(x_417) == 0) +{ +lean_object* x_418; +lean_dec(x_417); +lean_dec(x_415); +lean_dec(x_413); +lean_dec(x_411); +lean_dec(x_409); +lean_dec(x_391); +lean_dec(x_390); +lean_dec(x_389); +x_418 = lean_box(0); +return x_418; +} +else +{ +if (lean_obj_tag(x_391) == 9) +{ +lean_object* x_419; +x_419 = lean_ctor_get(x_391, 0); +lean_inc(x_419); +lean_dec(x_391); +if (lean_obj_tag(x_419) == 0) +{ +lean_object* x_420; +lean_dec(x_419); +lean_dec(x_417); +lean_dec(x_415); +lean_dec(x_413); +lean_dec(x_411); +lean_dec(x_409); +lean_dec(x_390); +lean_dec(x_389); +x_420 = lean_box(0); +return x_420; +} +else +{ +if (lean_obj_tag(x_390) == 9) +{ +lean_object* x_421; +x_421 = lean_ctor_get(x_390, 0); +lean_inc(x_421); +lean_dec(x_390); +if (lean_obj_tag(x_421) == 0) +{ +lean_object* x_422; +lean_dec(x_421); +lean_dec(x_419); +lean_dec(x_417); +lean_dec(x_415); +lean_dec(x_413); +lean_dec(x_411); +lean_dec(x_409); +lean_dec(x_389); +x_422 = lean_box(0); +return x_422; +} +else +{ +if (lean_obj_tag(x_389) == 9) +{ +lean_object* x_423; +x_423 = lean_ctor_get(x_389, 0); +lean_inc(x_423); +lean_dec(x_389); +if (lean_obj_tag(x_423) == 0) +{ +lean_object* x_424; +lean_dec(x_423); +lean_dec(x_421); +lean_dec(x_419); +lean_dec(x_417); +lean_dec(x_415); +lean_dec(x_413); +lean_dec(x_411); +lean_dec(x_409); +x_424 = lean_box(0); +return x_424; +} +else +{ +lean_object* x_425; lean_object* x_426; lean_object* x_427; lean_object* x_428; lean_object* x_429; lean_object* x_430; lean_object* x_431; uint8_t x_432; +x_425 = lean_ctor_get(x_409, 0); +lean_inc(x_425); +lean_dec(x_409); +x_426 = lean_ctor_get(x_411, 0); +lean_inc(x_426); +lean_dec(x_411); +x_427 = lean_ctor_get(x_413, 0); +lean_inc(x_427); +lean_dec(x_413); +x_428 = lean_ctor_get(x_415, 0); +lean_inc(x_428); +lean_dec(x_415); +x_429 = lean_ctor_get(x_417, 0); +lean_inc(x_429); +lean_dec(x_417); +x_430 = lean_ctor_get(x_419, 0); +lean_inc(x_430); +lean_dec(x_419); +x_431 = lean_ctor_get(x_421, 0); +lean_inc(x_431); +lean_dec(x_421); +x_432 = !lean_is_exclusive(x_423); +if (x_432 == 0) +{ +lean_object* x_433; lean_object* x_434; +x_433 = lean_ctor_get(x_423, 0); +x_434 = l_Lean_Name_mkStr8(x_425, x_426, x_427, x_428, x_429, x_430, x_431, x_433); +lean_ctor_set(x_423, 0, x_434); +return x_423; +} +else +{ +lean_object* x_435; lean_object* x_436; lean_object* x_437; +x_435 = lean_ctor_get(x_423, 0); +lean_inc(x_435); +lean_dec(x_423); +x_436 = l_Lean_Name_mkStr8(x_425, x_426, x_427, x_428, x_429, x_430, x_431, x_435); +x_437 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_437, 0, x_436); +return x_437; +} +} +} +else +{ +lean_object* x_438; +lean_dec(x_421); +lean_dec(x_419); +lean_dec(x_417); +lean_dec(x_415); +lean_dec(x_413); +lean_dec(x_411); +lean_dec(x_409); +lean_dec(x_389); +x_438 = lean_box(0); +return x_438; +} +} +} +else +{ +lean_object* x_439; +lean_dec(x_419); +lean_dec(x_417); +lean_dec(x_415); +lean_dec(x_413); +lean_dec(x_411); +lean_dec(x_409); +lean_dec(x_390); +lean_dec(x_389); +x_439 = lean_box(0); +return x_439; +} +} +} +else +{ +lean_object* x_440; +lean_dec(x_417); +lean_dec(x_415); +lean_dec(x_413); +lean_dec(x_411); +lean_dec(x_409); +lean_dec(x_391); +lean_dec(x_390); +lean_dec(x_389); +x_440 = lean_box(0); +return x_440; +} +} +} +else +{ +lean_object* x_441; +lean_dec(x_415); +lean_dec(x_413); +lean_dec(x_411); +lean_dec(x_409); +lean_dec(x_392); +lean_dec(x_391); +lean_dec(x_390); +lean_dec(x_389); +x_441 = lean_box(0); +return x_441; +} +} +} +else +{ +lean_object* x_442; +lean_dec(x_413); +lean_dec(x_411); +lean_dec(x_409); +lean_dec(x_393); +lean_dec(x_392); +lean_dec(x_391); +lean_dec(x_390); +lean_dec(x_389); +x_442 = lean_box(0); +return x_442; +} +} +} +else +{ +lean_object* x_443; +lean_dec(x_411); +lean_dec(x_409); +lean_dec(x_394); +lean_dec(x_393); +lean_dec(x_392); +lean_dec(x_391); +lean_dec(x_390); +lean_dec(x_389); +x_443 = lean_box(0); +return x_443; +} +} +} +else +{ +lean_object* x_444; +lean_dec(x_409); +lean_dec(x_395); +lean_dec(x_394); +lean_dec(x_393); +lean_dec(x_392); +lean_dec(x_391); +lean_dec(x_390); +lean_dec(x_389); +x_444 = lean_box(0); +return x_444; +} +} +} +else +{ +lean_object* x_445; +lean_dec(x_396); +lean_dec(x_395); +lean_dec(x_394); +lean_dec(x_393); +lean_dec(x_392); +lean_dec(x_391); +lean_dec(x_390); +lean_dec(x_389); +x_445 = lean_box(0); +return x_445; +} +} +} +} +} +else +{ +lean_object* x_446; +lean_dec(x_388); +lean_dec(x_387); +lean_dec(x_386); +lean_dec(x_385); +lean_dec(x_323); +lean_dec(x_267); +lean_dec(x_216); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_446 = lean_box(0); +return x_446; +} +} +else +{ +lean_object* x_447; +lean_dec(x_387); +lean_dec(x_386); +lean_dec(x_385); +lean_dec(x_323); +lean_dec(x_267); +lean_dec(x_216); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_447 = lean_box(0); +return x_447; +} +} +else +{ +lean_object* x_448; +lean_dec(x_386); +lean_dec(x_385); +lean_dec(x_323); +lean_dec(x_267); +lean_dec(x_216); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_448 = lean_box(0); +return x_448; +} +} +else +{ +lean_object* x_449; +lean_dec(x_385); +lean_dec(x_323); +lean_dec(x_267); +lean_dec(x_216); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_449 = lean_box(0); +return x_449; +} +} +else +{ +lean_object* x_450; +lean_dec(x_384); +lean_dec(x_323); +lean_dec(x_267); +lean_dec(x_216); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_450 = lean_box(0); +return x_450; +} +} +default: +{ +lean_object* x_451; +lean_dec(x_323); +lean_dec(x_267); +lean_dec(x_216); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_451 = lean_box(0); +return x_451; +} +} +} +default: +{ +lean_object* x_452; +lean_dec(x_267); +lean_dec(x_216); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_452 = lean_box(0); +return x_452; +} +} +} +default: +{ +lean_object* x_453; +lean_dec(x_216); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_453 = lean_box(0); +return x_453; +} +} +} +default: +{ +lean_object* x_454; +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_454 = lean_box(0); +return x_454; +} +} +} +default: +{ +lean_object* x_455; +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_455 = lean_box(0); +return x_455; +} +} +} +default: +{ +lean_object* x_456; +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_456 = lean_box(0); +return x_456; +} +} +} +default: +{ +lean_object* x_457; +lean_dec(x_23); +lean_dec(x_1); +x_457 = lean_box(0); +return x_457; +} +} +} +default: +{ +lean_object* x_458; +lean_dec(x_1); +x_458 = lean_box(0); +return x_458; +} +} +} +} lean_object* initialize_Lean_Environment(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Lean_Util_Recognizers(uint8_t builtin, lean_object* w) { @@ -1252,6 +4569,34 @@ l_Lean_Expr_prod_x3f___closed__1 = _init_l_Lean_Expr_prod_x3f___closed__1(); lean_mark_persistent(l_Lean_Expr_prod_x3f___closed__1); l_Lean_Expr_prod_x3f___closed__2 = _init_l_Lean_Expr_prod_x3f___closed__2(); lean_mark_persistent(l_Lean_Expr_prod_x3f___closed__2); +l_Lean_Expr_name_x3f___closed__1 = _init_l_Lean_Expr_name_x3f___closed__1(); +lean_mark_persistent(l_Lean_Expr_name_x3f___closed__1); +l_Lean_Expr_name_x3f___closed__2 = _init_l_Lean_Expr_name_x3f___closed__2(); +lean_mark_persistent(l_Lean_Expr_name_x3f___closed__2); +l_Lean_Expr_name_x3f___closed__3 = _init_l_Lean_Expr_name_x3f___closed__3(); +lean_mark_persistent(l_Lean_Expr_name_x3f___closed__3); +l_Lean_Expr_name_x3f___closed__4 = _init_l_Lean_Expr_name_x3f___closed__4(); +lean_mark_persistent(l_Lean_Expr_name_x3f___closed__4); +l_Lean_Expr_name_x3f___closed__5 = _init_l_Lean_Expr_name_x3f___closed__5(); +lean_mark_persistent(l_Lean_Expr_name_x3f___closed__5); +l_Lean_Expr_name_x3f___closed__6 = _init_l_Lean_Expr_name_x3f___closed__6(); +lean_mark_persistent(l_Lean_Expr_name_x3f___closed__6); +l_Lean_Expr_name_x3f___closed__7 = _init_l_Lean_Expr_name_x3f___closed__7(); +lean_mark_persistent(l_Lean_Expr_name_x3f___closed__7); +l_Lean_Expr_name_x3f___closed__8 = _init_l_Lean_Expr_name_x3f___closed__8(); +lean_mark_persistent(l_Lean_Expr_name_x3f___closed__8); +l_Lean_Expr_name_x3f___closed__9 = _init_l_Lean_Expr_name_x3f___closed__9(); +lean_mark_persistent(l_Lean_Expr_name_x3f___closed__9); +l_Lean_Expr_name_x3f___closed__10 = _init_l_Lean_Expr_name_x3f___closed__10(); +lean_mark_persistent(l_Lean_Expr_name_x3f___closed__10); +l_Lean_Expr_name_x3f___closed__11 = _init_l_Lean_Expr_name_x3f___closed__11(); +lean_mark_persistent(l_Lean_Expr_name_x3f___closed__11); +l_Lean_Expr_name_x3f___closed__12 = _init_l_Lean_Expr_name_x3f___closed__12(); +lean_mark_persistent(l_Lean_Expr_name_x3f___closed__12); +l_Lean_Expr_name_x3f___closed__13 = _init_l_Lean_Expr_name_x3f___closed__13(); +lean_mark_persistent(l_Lean_Expr_name_x3f___closed__13); +l_Lean_Expr_name_x3f___closed__14 = _init_l_Lean_Expr_name_x3f___closed__14(); +lean_mark_persistent(l_Lean_Expr_name_x3f___closed__14); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Lean/Widget/Diff.c b/stage0/stdlib/Lean/Widget/Diff.c index c6b7bb44d7a9..59c0361c0414 100644 --- a/stage0/stdlib/Lean/Widget/Diff.c +++ b/stage0/stdlib/Lean/Widget/Diff.c @@ -96,6 +96,7 @@ lean_object* l_Lean_Name_quickCmp___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_exprDiffCore___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_SavedState_restore(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_diffHypothesesBundle___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Widget_exprDiffCore___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Widget_diffInteractiveGoal___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_diffInteractiveGoals___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Widget_Diff_0__Lean_Widget_ExprDiffTag_noConfusion(lean_object*); @@ -117,7 +118,6 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_diffHypotheses_ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_diffInteractiveGoals___spec__3(uint8_t, lean_object*, uint8_t, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_RBNode_insert___at_Lean_MVarIdMap_insert___spec__1___rarg(lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_levelZero; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Widget_exprDiffCore___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Widget_diffHypothesesBundle_withTypeDiff___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_diffInteractiveGoals___spec__3___at_Lean_Widget_diffInteractiveGoals___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Widget_diffInteractiveGoal___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -145,6 +145,7 @@ static lean_object* l_Lean_Widget_initFn____x40_Lean_Widget_Diff___hyg_5____clos LEAN_EXPORT lean_object* l_Lean_RBNode_find___at_Lean_Widget_addDiffTags___spec__2___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_ExprDiff_insertAfterChange(lean_object*, uint8_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBMap_toList___at_Lean_Widget_instToStringExprDiff___spec__1(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Widget_exprDiffCore___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_ExprDiff_insertBeforeChange(lean_object*, uint8_t, lean_object*); static lean_object* l_Lean_Widget_diffHypothesesBundle_withTypeDiff___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_diffInteractiveGoals___spec__3___lambda__4(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -235,7 +236,6 @@ LEAN_EXPORT lean_object* l_Lean_Widget_diffInteractiveGoal___boxed(lean_object*, LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Widget_exprDiffCore___spec__3(lean_object*, size_t, size_t, lean_object*); uint8_t l_Lean_Exception_isRuntime(lean_object*); lean_object* l_List_toString___at_Lean_MetavarContext_MkBinding_instToStringException___spec__2(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Widget_exprDiffCore___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Widget_exprDiffCore___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_exprDiffCore___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_uset(lean_object*, size_t, lean_object*); @@ -4513,7 +4513,7 @@ return x_10; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Widget_exprDiffCore___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Widget_exprDiffCore___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { lean_object* x_15; uint8_t x_16; @@ -4732,7 +4732,7 @@ x_11 = l_Array_zip___rarg(x_1, x_2); x_12 = lean_array_get_size(x_11); x_13 = lean_mk_empty_array_with_capacity(x_12); x_14 = lean_unsigned_to_nat(0u); -x_15 = l_Array_mapIdxM_map___at_Lean_Widget_exprDiffCore___spec__2(x_3, x_4, x_1, x_11, x_11, x_12, x_14, lean_box(0), x_13, x_6, x_7, x_8, x_9, x_10); +x_15 = l_Array_mapFinIdxM_map___at_Lean_Widget_exprDiffCore___spec__2(x_3, x_4, x_1, x_11, x_11, x_12, x_14, lean_box(0), x_13, x_6, x_7, x_8, x_9, x_10); lean_dec(x_11); if (lean_obj_tag(x_15) == 0) { @@ -5765,11 +5765,11 @@ lean_dec(x_1); return x_11; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Widget_exprDiffCore___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Widget_exprDiffCore___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { lean_object* x_15; -x_15 = l_Array_mapIdxM_map___at_Lean_Widget_exprDiffCore___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +x_15 = l_Array_mapFinIdxM_map___at_Lean_Widget_exprDiffCore___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); diff --git a/stage0/stdlib/Lean/Widget/InteractiveCode.c b/stage0/stdlib/Lean/Widget/InteractiveCode.c index e3015469a58b..730fd3b47fa1 100644 --- a/stage0/stdlib/Lean/Widget/InteractiveCode.c +++ b/stage0/stdlib/Lean/Widget/InteractiveCode.c @@ -197,9 +197,9 @@ extern lean_object* l_Lean_Widget_instTypeNameInfoWithCtx; uint8_t lean_usize_dec_lt(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Widget_CodeWithInfos_mergePosMap(lean_object*, lean_object*); lean_object* lean_expr_dbg_to_string(lean_object*); -lean_object* l_List_bindTR_go___at___private_Lean_Data_Position_0__Lean_toJsonPosition____x40_Lean_Data_Position___hyg_237____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_CodeWithInfos_mergePosMap___rarg(lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_pp_mvars_anonymous; +lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Position_0__Lean_toJsonPosition____x40_Lean_Data_Position___hyg_237____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveCode___hyg_352____closed__2; LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveCode___hyg_352____lambda__1___boxed(lean_object*); static lean_object* l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveCode___hyg_352____closed__22; @@ -1472,7 +1472,7 @@ x_16 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_16, 0, x_8); lean_ctor_set(x_16, 1, x_15); x_17 = l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonDiffTag____x40_Lean_Widget_InteractiveCode___hyg_67____closed__1; -x_18 = l_List_bindTR_go___at___private_Lean_Data_Position_0__Lean_toJsonPosition____x40_Lean_Data_Position___hyg_237____spec__1(x_16, x_17); +x_18 = l_List_flatMapTR_go___at___private_Lean_Data_Position_0__Lean_toJsonPosition____x40_Lean_Data_Position___hyg_237____spec__1(x_16, x_17); x_19 = l_Lean_Json_mkObj(x_18); return x_19; } diff --git a/stage0/stdlib/Lean/Widget/InteractiveDiagnostic.c b/stage0/stdlib/Lean/Widget/InteractiveDiagnostic.c index a2d0cbbd5893..cf54a18ef54d 100644 --- a/stage0/stdlib/Lean/Widget/InteractiveDiagnostic.c +++ b/stage0/stdlib/Lean/Widget/InteractiveDiagnostic.c @@ -187,6 +187,7 @@ static lean_object* l_Lean_Widget_instInhabitedMsgEmbed___closed__2; static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1935____closed__10; static lean_object* l_Lean_Widget_InteractiveDiagnostic_toDiagnostic_prettyTt___lambda__1___closed__1; lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_instImpl____x40_Lean_Widget_InteractiveDiagnostic___hyg_547_; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodableDiagnosticWith_dec____x40_Lean_Widget_InteractiveDiagnostic___hyg_1850____spec__4___closed__2; LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_263_; @@ -220,7 +221,6 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodabl static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_766____lambda__2___closed__4; static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1935____closed__68; LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_766____lambda__3(lean_object*, lean_object*, lean_object*); -lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_766____lambda__1___closed__3; static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_go___closed__7; lean_object* l_Lean_Option_register___at_Lean_initFn____x40_Lean_Util_RecDepth___hyg_5____spec__1(lean_object*, lean_object*, lean_object*, lean_object*); @@ -6165,7 +6165,7 @@ x_40 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_40, 0, x_6); lean_ctor_set(x_40, 1, x_39); x_41 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_2476____closed__1; -x_42 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_40, x_41); +x_42 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_40, x_41); x_43 = l_Lean_Json_mkObj(x_42); return x_43; } diff --git a/stage0/stdlib/Lean/Widget/InteractiveGoal.c b/stage0/stdlib/Lean/Widget/InteractiveGoal.c index a63ef645c449..ee8de2e56998 100644 --- a/stage0/stdlib/Lean/Widget/InteractiveGoal.c +++ b/stage0/stdlib/Lean/Widget/InteractiveGoal.c @@ -188,6 +188,7 @@ static lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJ static lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoalCore_pretty___spec__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Widget_instAppendInteractiveGoals; static lean_object* l_Lean_Widget_instFromJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveGoal___hyg_657____closed__1; +lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveGoal___hyg_176____closed__3; static lean_object* l_Lean_Widget_withGoalCtx___rarg___lambda__2___closed__2; LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_Widget_instRpcEncodableInteractiveTermGoal_dec____x40_Lean_Widget_InteractiveGoal___hyg_2227____spec__1___boxed(lean_object*, lean_object*); @@ -218,7 +219,6 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_goalToInterac LEAN_EXPORT lean_object* l_Lean_PersistentArray_forIn___at_Lean_Widget_goalToInteractive___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Server_instRpcEncodableWithRpcRefOfTypeName_rpcEncode___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveGoal___hyg_3369____closed__7; -lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodableInteractiveTermGoal_enc____x40_Lean_Widget_InteractiveGoal___hyg_2227_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_withGoalCtx___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveGoal___hyg_1277____closed__23; @@ -1262,7 +1262,7 @@ x_37 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_37, 0, x_13); lean_ctor_set(x_37, 1, x_36); x_38 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveGoal___hyg_660____closed__1; -x_39 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_37, x_38); +x_39 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_37, x_38); x_40 = l_Lean_Json_mkObj(x_39); return x_40; } @@ -7312,7 +7312,7 @@ x_39 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_39, 0, x_13); lean_ctor_set(x_39, 1, x_38); x_40 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveGoal___hyg_660____closed__1; -x_41 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_39, x_40); +x_41 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_39, x_40); x_42 = l_Lean_Json_mkObj(x_41); return x_42; } @@ -10270,7 +10270,7 @@ x_27 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_27, 0, x_10); lean_ctor_set(x_27, 1, x_26); x_28 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveGoal___hyg_660____closed__1; -x_29 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_27, x_28); +x_29 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_27, x_28); x_30 = l_Lean_Json_mkObj(x_29); return x_30; } @@ -12002,7 +12002,7 @@ x_6 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_6, 0, x_5); lean_ctor_set(x_6, 1, x_4); x_7 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveGoal___hyg_660____closed__1; -x_8 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_6, x_7); +x_8 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_6, x_7); x_9 = l_Lean_Json_mkObj(x_8); return x_9; } diff --git a/stage0/stdlib/Lean/Widget/Types.c b/stage0/stdlib/Lean/Widget/Types.c index c65f357d95f8..22a8979d3241 100644 --- a/stage0/stdlib/Lean/Widget/Types.c +++ b/stage0/stdlib/Lean/Widget/Types.c @@ -35,6 +35,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Widget_Types_0__Lean_Widget_fromJsonRp static lean_object* l___private_Lean_Widget_Types_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_Types___hyg_62____closed__3; LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodableWidgetInstance_enc____x40_Lean_Widget_Types___hyg_3_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodableWidgetInstance_dec____x40_Lean_Widget_Types___hyg_3____lambda__1___boxed(lean_object*, lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Widget_instRpcEncodableWidgetInstance___closed__2; uint8_t lean_string_dec_eq(lean_object*, lean_object*); static lean_object* l___private_Lean_Widget_Types_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_Types___hyg_62____closed__7; @@ -72,7 +73,6 @@ LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodableWidgetInstance; LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_Types_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_Types___hyg_62____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_Widget_instRpcEncodableWidgetInstance_dec____x40_Lean_Widget_Types___hyg_3____spec__3(lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Widget_Types_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_Types___hyg_62____lambda__1(lean_object*); -lean_object* l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Widget_Types_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_Types___hyg_62____lambda__1___boxed(lean_object*); static lean_object* l___private_Lean_Widget_Types_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_Types___hyg_62____closed__35; LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodableWidgetInstance_dec____x40_Lean_Widget_Types___hyg_3_(lean_object*, lean_object*); @@ -583,7 +583,7 @@ x_17 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_17, 0, x_8); lean_ctor_set(x_17, 1, x_16); x_18 = l___private_Lean_Widget_Types_0__Lean_Widget_toJsonRpcEncodablePacket____x40_Lean_Widget_Types___hyg_261____closed__1; -x_19 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_17, x_18); +x_19 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_17, x_18); x_20 = l_Lean_Json_mkObj(x_19); return x_20; } diff --git a/stage0/stdlib/Lean/Widget/UserWidget.c b/stage0/stdlib/Lean/Widget/UserWidget.c index ffaa0ddb82fb..2a004760a5a1 100644 --- a/stage0/stdlib/Lean/Widget/UserWidget.c +++ b/stage0/stdlib/Lean/Widget/UserWidget.c @@ -352,6 +352,7 @@ lean_object* l_Lean_ScopedEnvExtension_modifyState___rarg(lean_object*, lean_obj lean_object* l_Lean_Name_append(lean_object*, lean_object*); static lean_object* l_Lean_Widget_addWidgetSpec___closed__7; LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Widget_elabShowPanelWidgetsCmd___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodableGetWidgetsResponse_enc____x40_Lean_Widget_UserWidget___hyg_4791____spec__1(size_t, size_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_elabShowPanelWidgetsCmd___spec__13___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Widget_elabShowPanelWidgetsCmd___spec__1___boxed(lean_object*, lean_object*); @@ -403,7 +404,6 @@ lean_object* l_Lean_bignumFromJson_x3f(lean_object*); static lean_object* l_Lean_Widget_addWidgetSpec___closed__1; static lean_object* l_Lean_Widget_showPanelWidgetsCmd___closed__9; static lean_object* l_Lean_Widget_instRpcEncodablePanelWidgetInstance___closed__3; -lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Widget_widgetInstanceSpec___closed__12; static lean_object* l_Lean_Widget_elabWidgetInstanceSpecAux___closed__46; static lean_object* l_Lean_Widget_instToJsonRpcEncodablePacket____x40_Lean_Widget_UserWidget___hyg_4536____closed__1; @@ -8210,7 +8210,7 @@ x_15 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_15, 0, x_8); lean_ctor_set(x_15, 1, x_14); x_16 = l_Lean_Widget_initFn____x40_Lean_Widget_UserWidget___hyg_240____lambda__4___closed__8; -x_17 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_15, x_16); +x_17 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_15, x_16); x_18 = l_Lean_Json_mkObj(x_17); return x_18; } @@ -8545,7 +8545,7 @@ x_7 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_7, 0, x_6); lean_ctor_set(x_7, 1, x_5); x_8 = l_Lean_Widget_initFn____x40_Lean_Widget_UserWidget___hyg_240____lambda__4___closed__8; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -18772,7 +18772,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_8); lean_ctor_set(x_14, 1, x_13); x_15 = l_Lean_Widget_initFn____x40_Lean_Widget_UserWidget___hyg_240____lambda__4___closed__8; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -18810,7 +18810,7 @@ x_30 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_30, 0, x_24); lean_ctor_set(x_30, 1, x_29); x_31 = l_Lean_Widget_initFn____x40_Lean_Widget_UserWidget___hyg_240____lambda__4___closed__8; -x_32 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_30, x_31); +x_32 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_30, x_31); x_33 = l_Lean_Json_mkObj(x_32); return x_33; } @@ -19848,7 +19848,7 @@ x_25 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_25, 0, x_10); lean_ctor_set(x_25, 1, x_24); x_26 = l_Lean_Widget_initFn____x40_Lean_Widget_UserWidget___hyg_240____lambda__4___closed__8; -x_27 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_25, x_26); +x_27 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_25, x_26); x_28 = l_Lean_Json_mkObj(x_27); return x_28; } @@ -21519,7 +21519,7 @@ x_6 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_6, 0, x_5); lean_ctor_set(x_6, 1, x_4); x_7 = l_Lean_Widget_initFn____x40_Lean_Widget_UserWidget___hyg_240____lambda__4___closed__8; -x_8 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_6, x_7); +x_8 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_6, x_7); x_9 = l_Lean_Json_mkObj(x_8); return x_9; } diff --git a/stage0/stdlib/Std/Data/DHashMap/Internal/Defs.c b/stage0/stdlib/Std/Data/DHashMap/Internal/Defs.c index e40f94a4f976..00fdd047a3c0 100644 --- a/stage0/stdlib/Std/Data/DHashMap/Internal/Defs.c +++ b/stage0/stdlib/Std/Data/DHashMap/Internal/Defs.c @@ -41,7 +41,6 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_get_x3f___rarg( LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_filterMap(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_insertManyUnit(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_getKey(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_bindTR_go___at_Std_DHashMap_Internal_toListModel___spec__1___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Std_DHashMap_Internal_Raw_u2080_expand_go___spec__1(lean_object*, lean_object*); lean_object* l_Nat_nextPowerOfTwo_go(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_get___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -56,6 +55,7 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_get_x21___rarg(lean_o LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_getKey_x21___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_getKey_x3f___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Std_DHashMap_Internal_Raw_u2080_filter___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at_Std_DHashMap_Internal_toListModel___spec__1___rarg___boxed(lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_filterMap___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Std_DHashMap_Internal_Raw_u2080_filter___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); @@ -81,6 +81,7 @@ lean_object* lean_array_to_list(lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_containsThenInsertIfNew(lean_object*, lean_object*); uint8_t l_Std_DHashMap_Internal_AssocList_contains___rarg(lean_object*, lean_object*, lean_object*); lean_object* l_Std_DHashMap_Internal_AssocList_getKey_x21___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at_Std_DHashMap_Internal_toListModel___spec__1___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_get___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_DHashMap_Internal_AssocList_getCast_x21___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_getThenInsertIfNew_x3f___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -115,7 +116,6 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expandIfNecessary___b static lean_object* l_Std_DHashMap_Internal_toListModel___rarg___closed__1; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_toListModel(lean_object*, lean_object*); lean_object* l_Std_DHashMap_Internal_AssocList_get_x21___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_bindTR_go___at_Std_DHashMap_Internal_toListModel___spec__1___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_get___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Defs_0__Std_DHashMap_Internal_numBucketsForCapacity(lean_object*); @@ -132,7 +132,6 @@ lean_object* lean_nat_sub(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_map___rarg(lean_object*, lean_object*); lean_object* lean_nat_mul(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_bindTR_go___at_Std_DHashMap_Internal_toListModel___spec__1(lean_object*, lean_object*); lean_object* l_List_foldl___at_Array_appendList___spec__1___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_empty(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_contains___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -151,6 +150,7 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_computeSize___rarg___boxed(lean LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(lean_object*, lean_object*); lean_object* lean_array_uget(lean_object*, size_t); size_t lean_array_size(lean_object*); +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at_Std_DHashMap_Internal_toListModel___spec__1(lean_object*, lean_object*); lean_object* l_Std_DHashMap_Internal_AssocList_getKey_x3f___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Std_DHashMap_Internal_Raw_u2080_filterMap___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Std_DHashMap_Internal_Raw_u2080_filter___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -192,7 +192,7 @@ lean_dec(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_List_bindTR_go___at_Std_DHashMap_Internal_toListModel___spec__1___rarg(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at_Std_DHashMap_Internal_toListModel___spec__1___rarg(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -214,11 +214,11 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_List_bindTR_go___at_Std_DHashMap_Internal_toListModel___spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at_Std_DHashMap_Internal_toListModel___spec__1(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_List_bindTR_go___at_Std_DHashMap_Internal_toListModel___spec__1___rarg___boxed), 2, 0); +x_3 = lean_alloc_closure((void*)(l_List_flatMapTR_go___at_Std_DHashMap_Internal_toListModel___spec__1___rarg___boxed), 2, 0); return x_3; } } @@ -237,7 +237,7 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_toListModel___rarg(lean_object* lean_object* x_2; lean_object* x_3; lean_object* x_4; x_2 = lean_array_to_list(x_1); x_3 = l_Std_DHashMap_Internal_toListModel___rarg___closed__1; -x_4 = l_List_bindTR_go___at_Std_DHashMap_Internal_toListModel___spec__1___rarg(x_2, x_3); +x_4 = l_List_flatMapTR_go___at_Std_DHashMap_Internal_toListModel___spec__1___rarg(x_2, x_3); lean_dec(x_2); return x_4; } @@ -250,11 +250,11 @@ x_3 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_toListModel___rarg), 1, return x_3; } } -LEAN_EXPORT lean_object* l_List_bindTR_go___at_Std_DHashMap_Internal_toListModel___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at_Std_DHashMap_Internal_toListModel___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_List_bindTR_go___at_Std_DHashMap_Internal_toListModel___spec__1___rarg(x_1, x_2); +x_3 = l_List_flatMapTR_go___at_Std_DHashMap_Internal_toListModel___spec__1___rarg(x_1, x_2); lean_dec(x_1); return x_3; } diff --git a/stage0/stdlib/Std/Sat/AIG.c b/stage0/stdlib/Std/Sat/AIG.c index 48e8ab51e33d..9af3dfc5dc70 100644 --- a/stage0/stdlib/Std/Sat/AIG.c +++ b/stage0/stdlib/Std/Sat/AIG.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG -// Imports: Init Std.Sat.AIG.Basic Std.Sat.AIG.LawfulOperator Std.Sat.AIG.Lemmas Std.Sat.AIG.Cached Std.Sat.AIG.CachedLemmas Std.Sat.AIG.CachedGates Std.Sat.AIG.CachedGatesLemmas Std.Sat.AIG.CNF Std.Sat.AIG.Relabel Std.Sat.AIG.RelabelNat Std.Sat.AIG.RefVec Std.Sat.AIG.RefVecOperator Std.Sat.AIG.LawfulVecOperator Std.Sat.AIG.If +// Imports: Std.Sat.AIG.Basic Std.Sat.AIG.LawfulOperator Std.Sat.AIG.Lemmas Std.Sat.AIG.Cached Std.Sat.AIG.CachedLemmas Std.Sat.AIG.CachedGates Std.Sat.AIG.CachedGatesLemmas Std.Sat.AIG.CNF Std.Sat.AIG.Relabel Std.Sat.AIG.RelabelNat Std.Sat.AIG.RefVec Std.Sat.AIG.RefVecOperator Std.Sat.AIG.LawfulVecOperator Std.Sat.AIG.If #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -13,7 +13,6 @@ #ifdef __cplusplus extern "C" { #endif -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_Basic(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_LawfulOperator(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_Lemmas(uint8_t builtin, lean_object*); @@ -33,9 +32,6 @@ LEAN_EXPORT lean_object* initialize_Std_Sat_AIG(uint8_t builtin, lean_object* w) lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Sat_AIG_Basic(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Sat/AIG/Basic.c b/stage0/stdlib/Std/Sat/AIG/Basic.c index 86f640dde9de..72649cf6f263 100644 --- a/stage0/stdlib/Std/Sat/AIG/Basic.c +++ b/stage0/stdlib/Std/Sat/AIG/Basic.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG.Basic -// Imports: Init Std.Data.HashMap Std.Data.HashSet +// Imports: Std.Data.HashMap Std.Data.HashSet #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -5655,7 +5655,6 @@ lean_dec(x_1); return x_6; } } -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Data_HashMap(uint8_t builtin, lean_object*); lean_object* initialize_Std_Data_HashSet(uint8_t builtin, lean_object*); static bool _G_initialized = false; @@ -5663,9 +5662,6 @@ LEAN_EXPORT lean_object* initialize_Std_Sat_AIG_Basic(uint8_t builtin, lean_obje lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Data_HashMap(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Sat/AIG/CNF.c b/stage0/stdlib/Std/Sat/AIG/CNF.c index 63086e18047d..f2d7121e4c44 100644 --- a/stage0/stdlib/Std/Sat/AIG/CNF.c +++ b/stage0/stdlib/Std/Sat/AIG/CNF.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG.CNF -// Imports: Init Std.Sat.CNF Std.Sat.AIG.Basic Std.Sat.AIG.Lemmas +// Imports: Std.Sat.CNF Std.Sat.AIG.Basic Std.Sat.AIG.Lemmas #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -1063,7 +1063,6 @@ x_15 = l_Std_Sat_CNF_relabel___rarg(x_14, x_13); return x_15; } } -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_CNF(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_Basic(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_Lemmas(uint8_t builtin, lean_object*); @@ -1072,9 +1071,6 @@ LEAN_EXPORT lean_object* initialize_Std_Sat_AIG_CNF(uint8_t builtin, lean_object lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Sat_CNF(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Sat/AIG/Cached.c b/stage0/stdlib/Std/Sat/AIG/Cached.c index 69bee4045bfe..13918a403087 100644 --- a/stage0/stdlib/Std/Sat/AIG/Cached.c +++ b/stage0/stdlib/Std/Sat/AIG/Cached.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG.Cached -// Imports: Init Std.Sat.AIG.Basic Std.Sat.AIG.Lemmas +// Imports: Std.Sat.AIG.Basic Std.Sat.AIG.Lemmas #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -1467,7 +1467,6 @@ x_2 = lean_alloc_closure((void*)(l_Std_Sat_AIG_mkGateCached___rarg), 4, 0); return x_2; } } -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_Basic(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_Lemmas(uint8_t builtin, lean_object*); static bool _G_initialized = false; @@ -1475,9 +1474,6 @@ LEAN_EXPORT lean_object* initialize_Std_Sat_AIG_Cached(uint8_t builtin, lean_obj lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Sat_AIG_Basic(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Sat/AIG/CachedGates.c b/stage0/stdlib/Std/Sat/AIG/CachedGates.c index 1ac889fdd5bd..8cc4869a66e8 100644 --- a/stage0/stdlib/Std/Sat/AIG/CachedGates.c +++ b/stage0/stdlib/Std/Sat/AIG/CachedGates.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG.CachedGates -// Imports: Init Std.Sat.AIG.Cached Std.Sat.AIG.CachedLemmas +// Imports: Std.Sat.AIG.Cached Std.Sat.AIG.CachedLemmas #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -646,7 +646,6 @@ x_2 = lean_alloc_closure((void*)(l_Std_Sat_AIG_mkImpCached___rarg), 4, 0); return x_2; } } -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_Cached(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_CachedLemmas(uint8_t builtin, lean_object*); static bool _G_initialized = false; @@ -654,9 +653,6 @@ LEAN_EXPORT lean_object* initialize_Std_Sat_AIG_CachedGates(uint8_t builtin, lea lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Sat_AIG_Cached(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Sat/AIG/CachedGatesLemmas.c b/stage0/stdlib/Std/Sat/AIG/CachedGatesLemmas.c index 460546e61625..f99ec336c349 100644 --- a/stage0/stdlib/Std/Sat/AIG/CachedGatesLemmas.c +++ b/stage0/stdlib/Std/Sat/AIG/CachedGatesLemmas.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG.CachedGatesLemmas -// Imports: Init Std.Sat.AIG.CachedGates Std.Sat.AIG.LawfulOperator +// Imports: Std.Sat.AIG.CachedGates Std.Sat.AIG.LawfulOperator #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -13,7 +13,6 @@ #ifdef __cplusplus extern "C" { #endif -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_CachedGates(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_LawfulOperator(uint8_t builtin, lean_object*); static bool _G_initialized = false; @@ -21,9 +20,6 @@ LEAN_EXPORT lean_object* initialize_Std_Sat_AIG_CachedGatesLemmas(uint8_t builti lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Sat_AIG_CachedGates(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Sat/AIG/CachedLemmas.c b/stage0/stdlib/Std/Sat/AIG/CachedLemmas.c index b881f69cee64..faf22391fc17 100644 --- a/stage0/stdlib/Std/Sat/AIG/CachedLemmas.c +++ b/stage0/stdlib/Std/Sat/AIG/CachedLemmas.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG.CachedLemmas -// Imports: Init Std.Sat.AIG.Cached +// Imports: Std.Sat.AIG.Cached #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -889,16 +889,12 @@ lean_dec(x_2); return x_5; } } -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_Cached(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Std_Sat_AIG_CachedLemmas(uint8_t builtin, lean_object* w) { lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Sat_AIG_Cached(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Sat/AIG/If.c b/stage0/stdlib/Std/Sat/AIG/If.c index 8be164b60daf..e897651b0000 100644 --- a/stage0/stdlib/Std/Sat/AIG/If.c +++ b/stage0/stdlib/Std/Sat/AIG/If.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG.If -// Imports: Init Std.Sat.AIG.CachedGatesLemmas Std.Sat.AIG.LawfulVecOperator +// Imports: Std.Sat.AIG.CachedGatesLemmas Std.Sat.AIG.LawfulVecOperator #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -201,7 +201,6 @@ lean_dec(x_3); return x_6; } } -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_CachedGatesLemmas(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_LawfulVecOperator(uint8_t builtin, lean_object*); static bool _G_initialized = false; @@ -209,9 +208,6 @@ LEAN_EXPORT lean_object* initialize_Std_Sat_AIG_If(uint8_t builtin, lean_object* lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Sat_AIG_CachedGatesLemmas(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Sat/AIG/LawfulOperator.c b/stage0/stdlib/Std/Sat/AIG/LawfulOperator.c index d2d551df2813..4aff9ce69d6b 100644 --- a/stage0/stdlib/Std/Sat/AIG/LawfulOperator.c +++ b/stage0/stdlib/Std/Sat/AIG/LawfulOperator.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG.LawfulOperator -// Imports: Init Std.Sat.AIG.Basic +// Imports: Std.Sat.AIG.Basic #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -69,16 +69,12 @@ x_3 = lean_alloc_closure((void*)(l___private_Std_Sat_AIG_LawfulOperator_0__Std_S return x_3; } } -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_Basic(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Std_Sat_AIG_LawfulOperator(uint8_t builtin, lean_object* w) { lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Sat_AIG_Basic(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Sat/AIG/LawfulVecOperator.c b/stage0/stdlib/Std/Sat/AIG/LawfulVecOperator.c index 50228c352eff..2c72608b1ba9 100644 --- a/stage0/stdlib/Std/Sat/AIG/LawfulVecOperator.c +++ b/stage0/stdlib/Std/Sat/AIG/LawfulVecOperator.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG.LawfulVecOperator -// Imports: Init Std.Sat.AIG.LawfulOperator Std.Sat.AIG.RefVec +// Imports: Std.Sat.AIG.LawfulOperator Std.Sat.AIG.RefVec #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -13,7 +13,6 @@ #ifdef __cplusplus extern "C" { #endif -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_LawfulOperator(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_RefVec(uint8_t builtin, lean_object*); static bool _G_initialized = false; @@ -21,9 +20,6 @@ LEAN_EXPORT lean_object* initialize_Std_Sat_AIG_LawfulVecOperator(uint8_t builti lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Sat_AIG_LawfulOperator(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Sat/AIG/Lemmas.c b/stage0/stdlib/Std/Sat/AIG/Lemmas.c index a06c3e522032..35bf19ddd042 100644 --- a/stage0/stdlib/Std/Sat/AIG/Lemmas.c +++ b/stage0/stdlib/Std/Sat/AIG/Lemmas.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG.Lemmas -// Imports: Init Std.Sat.AIG.Basic Std.Sat.AIG.LawfulOperator +// Imports: Std.Sat.AIG.Basic Std.Sat.AIG.LawfulOperator #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -69,7 +69,6 @@ x_3 = lean_alloc_closure((void*)(l___private_Std_Sat_AIG_Lemmas_0__Std_Sat_AIG_t return x_3; } } -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_Basic(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_LawfulOperator(uint8_t builtin, lean_object*); static bool _G_initialized = false; @@ -77,9 +76,6 @@ LEAN_EXPORT lean_object* initialize_Std_Sat_AIG_Lemmas(uint8_t builtin, lean_obj lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Sat_AIG_Basic(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Sat/AIG/RefVec.c b/stage0/stdlib/Std/Sat/AIG/RefVec.c index 845de5f3c0c9..c41cb32b11e9 100644 --- a/stage0/stdlib/Std/Sat/AIG/RefVec.c +++ b/stage0/stdlib/Std/Sat/AIG/RefVec.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG.RefVec -// Imports: Init Std.Sat.AIG.LawfulOperator Std.Sat.AIG.CachedGatesLemmas +// Imports: Std.Sat.AIG.LawfulOperator Std.Sat.AIG.CachedGatesLemmas #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -591,7 +591,6 @@ lean_dec(x_2); return x_7; } } -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_LawfulOperator(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_CachedGatesLemmas(uint8_t builtin, lean_object*); static bool _G_initialized = false; @@ -599,9 +598,6 @@ LEAN_EXPORT lean_object* initialize_Std_Sat_AIG_RefVec(uint8_t builtin, lean_obj lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Sat_AIG_LawfulOperator(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Sat/AIG/RefVecOperator.c b/stage0/stdlib/Std/Sat/AIG/RefVecOperator.c index 61c8d0cba16b..153a72172d92 100644 --- a/stage0/stdlib/Std/Sat/AIG/RefVecOperator.c +++ b/stage0/stdlib/Std/Sat/AIG/RefVecOperator.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG.RefVecOperator -// Imports: Init Std.Sat.AIG.RefVecOperator.Map Std.Sat.AIG.RefVecOperator.Zip Std.Sat.AIG.RefVecOperator.Fold +// Imports: Std.Sat.AIG.RefVecOperator.Map Std.Sat.AIG.RefVecOperator.Zip Std.Sat.AIG.RefVecOperator.Fold #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -13,7 +13,6 @@ #ifdef __cplusplus extern "C" { #endif -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_RefVecOperator_Map(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_RefVecOperator_Zip(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_RefVecOperator_Fold(uint8_t builtin, lean_object*); @@ -22,9 +21,6 @@ LEAN_EXPORT lean_object* initialize_Std_Sat_AIG_RefVecOperator(uint8_t builtin, lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Sat_AIG_RefVecOperator_Map(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Sat/AIG/RefVecOperator/Fold.c b/stage0/stdlib/Std/Sat/AIG/RefVecOperator/Fold.c index 31a1388f8f0e..ecf2d343b603 100644 --- a/stage0/stdlib/Std/Sat/AIG/RefVecOperator/Fold.c +++ b/stage0/stdlib/Std/Sat/AIG/RefVecOperator/Fold.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG.RefVecOperator.Fold -// Imports: Init Std.Sat.AIG.RefVec Std.Sat.AIG.LawfulVecOperator +// Imports: Std.Sat.AIG.RefVec Std.Sat.AIG.LawfulVecOperator #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -154,7 +154,6 @@ x_2 = lean_alloc_closure((void*)(l_Std_Sat_AIG_RefVec_fold___rarg), 4, 0); return x_2; } } -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_RefVec(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_LawfulVecOperator(uint8_t builtin, lean_object*); static bool _G_initialized = false; @@ -162,9 +161,6 @@ LEAN_EXPORT lean_object* initialize_Std_Sat_AIG_RefVecOperator_Fold(uint8_t buil lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Sat_AIG_RefVec(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Sat/AIG/RefVecOperator/Map.c b/stage0/stdlib/Std/Sat/AIG/RefVecOperator/Map.c index 86eb7cbc0324..72ad864a69be 100644 --- a/stage0/stdlib/Std/Sat/AIG/RefVecOperator/Map.c +++ b/stage0/stdlib/Std/Sat/AIG/RefVecOperator/Map.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG.RefVecOperator.Map -// Imports: Init Std.Sat.AIG.RefVec Std.Sat.AIG.LawfulVecOperator +// Imports: Std.Sat.AIG.RefVec Std.Sat.AIG.LawfulVecOperator #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -119,7 +119,6 @@ lean_dec(x_1); return x_6; } } -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_RefVec(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_LawfulVecOperator(uint8_t builtin, lean_object*); static bool _G_initialized = false; @@ -127,9 +126,6 @@ LEAN_EXPORT lean_object* initialize_Std_Sat_AIG_RefVecOperator_Map(uint8_t built lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Sat_AIG_RefVec(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Sat/AIG/RefVecOperator/Zip.c b/stage0/stdlib/Std/Sat/AIG/RefVecOperator/Zip.c index 7325781cbe0f..370cc8eec26c 100644 --- a/stage0/stdlib/Std/Sat/AIG/RefVecOperator/Zip.c +++ b/stage0/stdlib/Std/Sat/AIG/RefVecOperator/Zip.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG.RefVecOperator.Zip -// Imports: Init Std.Sat.AIG.RefVec Std.Sat.AIG.LawfulVecOperator +// Imports: Std.Sat.AIG.RefVec Std.Sat.AIG.LawfulVecOperator #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -130,7 +130,6 @@ lean_dec(x_1); return x_6; } } -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_RefVec(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_LawfulVecOperator(uint8_t builtin, lean_object*); static bool _G_initialized = false; @@ -138,9 +137,6 @@ LEAN_EXPORT lean_object* initialize_Std_Sat_AIG_RefVecOperator_Zip(uint8_t built lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Sat_AIG_RefVec(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Sat/AIG/Relabel.c b/stage0/stdlib/Std/Sat/AIG/Relabel.c index c80b596fb6f9..e8df5069f458 100644 --- a/stage0/stdlib/Std/Sat/AIG/Relabel.c +++ b/stage0/stdlib/Std/Sat/AIG/Relabel.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG.Relabel -// Imports: Init Std.Sat.AIG.Basic Std.Sat.AIG.Lemmas +// Imports: Std.Sat.AIG.Basic Std.Sat.AIG.Lemmas #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -322,7 +322,6 @@ lean_dec(x_2); return x_5; } } -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_Basic(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_Lemmas(uint8_t builtin, lean_object*); static bool _G_initialized = false; @@ -330,9 +329,6 @@ LEAN_EXPORT lean_object* initialize_Std_Sat_AIG_Relabel(uint8_t builtin, lean_ob lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Sat_AIG_Basic(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Sat/AIG/RelabelNat.c b/stage0/stdlib/Std/Sat/AIG/RelabelNat.c index 69c74ae44184..9ccfa74c6d26 100644 --- a/stage0/stdlib/Std/Sat/AIG/RelabelNat.c +++ b/stage0/stdlib/Std/Sat/AIG/RelabelNat.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG.RelabelNat -// Imports: Init Std.Sat.AIG.Relabel +// Imports: Std.Sat.AIG.Relabel #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -1377,16 +1377,12 @@ x_2 = lean_alloc_closure((void*)(l_Std_Sat_AIG_Entrypoint_relabelNat___rarg), 3, return x_2; } } -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_Relabel(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Std_Sat_AIG_RelabelNat(uint8_t builtin, lean_object* w) { lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Sat_AIG_Relabel(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Tactic/BVDecide/Bitblast/BVExpr/Basic.c b/stage0/stdlib/Std/Tactic/BVDecide/Bitblast/BVExpr/Basic.c index 781ddf21532e..f8aeed3c0237 100644 --- a/stage0/stdlib/Std/Tactic/BVDecide/Bitblast/BVExpr/Basic.c +++ b/stage0/stdlib/Std/Tactic/BVDecide/Bitblast/BVExpr/Basic.c @@ -78,6 +78,7 @@ static lean_object* l_Std_Tactic_BVDecide_BVExpr_toString___closed__9; static lean_object* l_Std_Tactic_BVDecide_BVExpr_toString___closed__4; static lean_object* l___private_Std_Tactic_BVDecide_Bitblast_BVExpr_Basic_0__Std_Tactic_BVDecide_reprBVBit____x40_Std_Tactic_BVDecide_Bitblast_BVExpr_Basic___hyg_287____closed__2; static lean_object* l_Std_Tactic_BVDecide_BVUnOp_toString___closed__7; +lean_object* l_BitVec_sdiv(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Std_Tactic_BVDecide_Bitblast_BVExpr_Basic_0__Std_Tactic_BVDecide_reprBVBit____x40_Std_Tactic_BVDecide_Bitblast_BVExpr_Basic___hyg_287____closed__4; LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVBinOp_eval(lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_instDecidableEqBVBit___boxed(lean_object*, lean_object*); @@ -147,6 +148,7 @@ lean_object* lean_string_append(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_Assignment_getD___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_toString(lean_object*, lean_object*); static lean_object* l_Std_Tactic_BVDecide_BVBinOp_toString___closed__5; +static lean_object* l_Std_Tactic_BVDecide_BVBinOp_toString___closed__8; static lean_object* l___private_Std_Tactic_BVDecide_Bitblast_BVExpr_Basic_0__Std_Tactic_BVDecide_reprBVBit____x40_Std_Tactic_BVDecide_Bitblast_BVExpr_Basic___hyg_287____closed__18; LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_instHashableBVBit; LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_instToStringBVBit(lean_object*); @@ -684,12 +686,18 @@ lean_object* x_7; x_7 = lean_unsigned_to_nat(5u); return x_7; } -default: +case 6: { lean_object* x_8; x_8 = lean_unsigned_to_nat(6u); return x_8; } +default: +{ +lean_object* x_9; +x_9 = lean_unsigned_to_nat(7u); +return x_9; +} } } } @@ -811,6 +819,14 @@ x_1 = lean_mk_string_unchecked("%ᵤ", 4, 2); return x_1; } } +static lean_object* _init_l_Std_Tactic_BVDecide_BVBinOp_toString___closed__8() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("/ₛ", 4, 2); +return x_1; +} +} LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVBinOp_toString(uint8_t x_1) { _start: { @@ -851,12 +867,18 @@ lean_object* x_7; x_7 = l_Std_Tactic_BVDecide_BVBinOp_toString___closed__6; return x_7; } -default: +case 6: { lean_object* x_8; x_8 = l_Std_Tactic_BVDecide_BVBinOp_toString___closed__7; return x_8; } +default: +{ +lean_object* x_9; +x_9 = l_Std_Tactic_BVDecide_BVBinOp_toString___closed__8; +return x_9; +} } } } @@ -926,12 +948,18 @@ lean_object* x_10; x_10 = lean_nat_div(x_3, x_4); return x_10; } -default: +case 6: { lean_object* x_11; x_11 = lean_nat_mod(x_3, x_4); return x_11; } +default: +{ +lean_object* x_12; +x_12 = l_BitVec_sdiv(x_1, x_3, x_4); +return x_12; +} } } } @@ -2192,6 +2220,8 @@ l_Std_Tactic_BVDecide_BVBinOp_toString___closed__6 = _init_l_Std_Tactic_BVDecide lean_mark_persistent(l_Std_Tactic_BVDecide_BVBinOp_toString___closed__6); l_Std_Tactic_BVDecide_BVBinOp_toString___closed__7 = _init_l_Std_Tactic_BVDecide_BVBinOp_toString___closed__7(); lean_mark_persistent(l_Std_Tactic_BVDecide_BVBinOp_toString___closed__7); +l_Std_Tactic_BVDecide_BVBinOp_toString___closed__8 = _init_l_Std_Tactic_BVDecide_BVBinOp_toString___closed__8(); +lean_mark_persistent(l_Std_Tactic_BVDecide_BVBinOp_toString___closed__8); l_Std_Tactic_BVDecide_BVBinOp_instToString___closed__1 = _init_l_Std_Tactic_BVDecide_BVBinOp_instToString___closed__1(); lean_mark_persistent(l_Std_Tactic_BVDecide_BVBinOp_instToString___closed__1); l_Std_Tactic_BVDecide_BVBinOp_instToString = _init_l_Std_Tactic_BVDecide_BVBinOp_instToString(); diff --git a/stage0/stdlib/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Impl/Expr.c b/stage0/stdlib/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Impl/Expr.c index ec8728ccd3d9..171fdd68eb70 100644 --- a/stage0/stdlib/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Impl/Expr.c +++ b/stage0/stdlib/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Impl/Expr.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Expr -// Imports: Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Var Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Const Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Not Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.ShiftLeft Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.ShiftRight Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Add Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.ZeroExtend Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Append Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Replicate Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Extract Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.RotateLeft Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.RotateRight Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.SignExtend Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Mul Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Udiv Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Umod +// Imports: Init.Data.AC Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Var Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Const Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Not Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.ShiftLeft Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.ShiftRight Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Add Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.ZeroExtend Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Append Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Replicate Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Extract Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.RotateLeft Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.RotateRight Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.SignExtend Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Mul Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Udiv Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Umod Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Sdiv #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -13,116 +13,119 @@ #ifdef __cplusplus extern "C" { #endif -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateRight___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__28___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__42(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastReplicate___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__33___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastReplicate___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__35___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastArithShiftRightConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__32___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__39(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Sat_AIG_RefVec_map___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__18(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateRight___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__28(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__42___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastArithShiftRightConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__32(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__44(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastNot___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__17___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Sat_AIG_RefVec_zip___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__5___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRightConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__26___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastArithShiftRightConst_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__33___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); lean_object* l_Std_Sat_AIG_RefVec_ite___at_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul_go___spec__27(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Sat_AIG_RefVec_zip___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__5(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSignExtend___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__35___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateRight_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__31(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSignExtend___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__37___boxed(lean_object*, lean_object*, lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); lean_object* l_Std_Sat_AIG_mkAndCached___at_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul_go___spec__25(lean_object*, lean_object*); lean_object* l_Std_Sat_AIG_mkConstCached___at_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul_go___spec__4(lean_object*, uint8_t); lean_object* l_Std_Sat_AIG_mkOrCached___at_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul_go___spec__26(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateLeft_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__27___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_mkOverflowBit_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__22___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_go___closed__1; LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_mkOverflowBit___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__21(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastNot___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__17(lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_go___closed__2; +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight_twoPowShift___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__43___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVPred_mkEq___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__8(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Sat_AIG_RefVec_fold___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__10(lean_object*, lean_object*); lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul_blast___spec__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__41___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv_blastShiftConcat___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__14___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Std_Sat_AIG_mkNotCached___at_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul_go___spec__30(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv_blastShiftConcat___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__14(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastAppend___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__32(lean_object*, lean_object*, lean_object*); lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastAdd___at_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul_go___spec__16(lean_object*, lean_object*, lean_object*); lean_object* l_Std_Sat_AIG_mkXorCached___at_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul_go___spec__20(lean_object*, lean_object*); lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeftConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul_go___spec__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Tactic_BVDecide_BVPred_mkEq___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__8___closed__1; -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastArithShiftRightConst_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__31(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__40___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastArithShiftRightConst_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__33(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__42(lean_object*, lean_object*, lean_object*); lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastVar(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Sat_AIG_RefVec_fold_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__37___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv_blastDivSubtractShift___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRightConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__26(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Sat_AIG_RefVec_fold_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateLeft___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__26___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv_signBranch___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__25(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_go(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Sat_AIG_RefVec_zip_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___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_Std_Tactic_BVDecide_BVExpr_bitblast_blastSub___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__15(lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Tactic_BVDecide_BVPred_mkEq___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__8___closed__2; +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft_twoPowShift___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__40(lean_object*, lean_object*, lean_object*); lean_object* l_BitVec_ofNat(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv_blastDivSubtractShift___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___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_Std_Tactic_BVDecide_BVExpr_bitblast_blastArithShiftRightConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__30___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateLeft_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__29(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSignExtend___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__37(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVPred_mkUlt___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__20(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastZeroExtend___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_mkOverflowBit_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__22(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateLeft_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__27(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastReplicate___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__33(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastAppend___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__32___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSignExtend_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__38(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast(lean_object*, lean_object*, lean_object*); lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_mkFullAdderCarry___at_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul_go___spec__24(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateLeft_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__29___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_Tactic_BVDecide_instDecidableEqBVBit___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastNeg___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__16___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastReplicate_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__34(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRightConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__24(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastReplicate_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__36(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__44___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Sat_AIG_RefVec_map_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__19(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastNot___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__17___closed__1; -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRightConst_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__25(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSignExtend_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__36___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__42___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastReplicate_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__36___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastExtract_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__4(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_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__39___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastZeroExtend_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUmod___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__23(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft_twoPowShift___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__40___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight_twoPowShift___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__41(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSignExtend___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__35(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateLeft___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__28___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastExtract_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_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_Std_Tactic_BVDecide_BVExpr_bitblast_blastZeroExtend_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__2___closed__1; lean_object* lean_nat_pow(lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__24(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRightConst_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__27(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_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft_twoPowShift___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__38(lean_object*, lean_object*, lean_object*); lean_object* lean_nat_mod(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastZeroExtend_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__39(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRightConst_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__27___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Sat_AIG_RefVec_map___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__18___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateLeft___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__26(lean_object*, lean_object*, lean_object*); lean_object* l_Std_Sat_AIG_mkGateCached___at_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul_go___spec__21(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastArithShiftRightConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__30(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRightConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__24___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateLeft___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__28(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastExtract___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__3(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__39___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateRight___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__30___boxed(lean_object*, lean_object*, lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateRight_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__29(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__37(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft_twoPowShift___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__38___boxed(lean_object*, lean_object*, lean_object*); lean_object* lean_nat_mul(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastNeg___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__16(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateRight___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__30(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastAppend___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__34(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastReplicate___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__35(lean_object*, lean_object*, lean_object*); lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastArithShiftRightConst_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__31___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateRight_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__29___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRightConst_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__25___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSignExtend_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__36(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__40(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv_signBranch___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__25___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSignExtend_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__38___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__7(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight_twoPowShift___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__41___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateRight_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__31___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastAppend___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__34___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSub___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__15___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Sat_AIG_RefVec_zip_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_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_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastZeroExtend___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Sat_AIG_mkBEqCached___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__9(lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastExtract___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__3___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__41(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_Sat_AIG_RefVec_empty___at_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul_go___spec__2(lean_object*); -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastReplicate_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__34___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight_twoPowShift___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__43(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Sat_AIG_RefVec_map_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__19___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* _init_l_Std_Tactic_BVDecide_BVExpr_bitblast_blastZeroExtend_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__2___closed__1() { _start: @@ -1466,7 +1469,350 @@ return x_43; } } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRightConst_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___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_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv_signBranch___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__25(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_4 = lean_ctor_get(x_3, 0); +x_5 = lean_ctor_get(x_3, 1); +x_6 = lean_ctor_get(x_3, 2); +x_7 = lean_ctor_get(x_3, 3); +x_8 = lean_ctor_get(x_3, 4); +x_9 = lean_ctor_get(x_3, 5); +x_10 = lean_ctor_get(x_3, 6); +x_11 = lean_unsigned_to_nat(1u); +x_12 = lean_nat_sub(x_4, x_11); +x_13 = lean_array_fget(x_6, x_12); +x_14 = lean_array_fget(x_5, x_12); +lean_dec(x_12); +lean_inc(x_7); +lean_inc(x_8); +lean_inc(x_13); +x_15 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_15, 0, x_13); +lean_ctor_set(x_15, 1, x_8); +lean_ctor_set(x_15, 2, x_7); +x_16 = l_Std_Sat_AIG_RefVec_ite___at_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul_go___spec__27(x_1, x_2, x_15); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +lean_inc(x_9); +lean_inc(x_10); +x_19 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_19, 0, x_13); +lean_ctor_set(x_19, 1, x_10); +lean_ctor_set(x_19, 2, x_9); +x_20 = l_Std_Sat_AIG_RefVec_ite___at_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul_go___spec__27(x_1, x_17, x_19); +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +x_23 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_23, 0, x_14); +lean_ctor_set(x_23, 1, x_22); +lean_ctor_set(x_23, 2, x_18); +x_24 = l_Std_Sat_AIG_RefVec_ite___at_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul_go___spec__27(x_1, x_21, x_23); +return x_24; +} +} +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__24(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_1, x_4); +if (x_5 == 0) +{ +uint8_t x_6; +x_6 = !lean_is_exclusive(x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_7 = lean_ctor_get(x_3, 0); +x_8 = lean_ctor_get(x_3, 1); +lean_inc(x_7); +x_9 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastNeg___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__16(x_1, x_2, x_7); +x_10 = lean_ctor_get(x_9, 0); +lean_inc(x_10); +x_11 = lean_ctor_get(x_9, 1); +lean_inc(x_11); +lean_dec(x_9); +lean_inc(x_8); +x_12 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastNeg___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__16(x_1, x_10, x_8); +x_13 = !lean_is_exclusive(x_12); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_14 = lean_ctor_get(x_12, 0); +x_15 = lean_ctor_get(x_12, 1); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_1); +x_16 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__7(x_1, x_14, x_3); +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); +lean_inc(x_7); +lean_ctor_set(x_12, 0, x_7); +lean_inc(x_1); +x_19 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__7(x_1, x_17, x_12); +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_Std_Tactic_BVDecide_BVExpr_bitblast_blastNeg___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__16(x_1, x_20, 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); +lean_inc(x_8); +lean_inc(x_11); +x_25 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_25, 0, x_11); +lean_ctor_set(x_25, 1, x_8); +lean_inc(x_1); +x_26 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__7(x_1, x_23, x_25); +x_27 = lean_ctor_get(x_26, 0); +lean_inc(x_27); +x_28 = lean_ctor_get(x_26, 1); +lean_inc(x_28); +lean_dec(x_26); +x_29 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastNeg___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__16(x_1, x_27, 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); +lean_dec(x_29); +x_32 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_32, 0, x_11); +lean_ctor_set(x_32, 1, x_15); +lean_inc(x_1); +x_33 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__7(x_1, x_30, 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); +lean_inc(x_1); +x_36 = lean_alloc_ctor(0, 7, 0); +lean_ctor_set(x_36, 0, x_1); +lean_ctor_set(x_36, 1, x_7); +lean_ctor_set(x_36, 2, x_8); +lean_ctor_set(x_36, 3, x_18); +lean_ctor_set(x_36, 4, x_24); +lean_ctor_set(x_36, 5, x_31); +lean_ctor_set(x_36, 6, x_35); +x_37 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv_signBranch___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__25(x_1, x_34, x_36); +lean_dec(x_36); +lean_dec(x_1); +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; 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_38 = lean_ctor_get(x_12, 0); +x_39 = lean_ctor_get(x_12, 1); +lean_inc(x_39); +lean_inc(x_38); +lean_dec(x_12); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_1); +x_40 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__7(x_1, x_38, x_3); +x_41 = lean_ctor_get(x_40, 0); +lean_inc(x_41); +x_42 = lean_ctor_get(x_40, 1); +lean_inc(x_42); +lean_dec(x_40); +lean_inc(x_39); +lean_inc(x_7); +x_43 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_43, 0, x_7); +lean_ctor_set(x_43, 1, x_39); +lean_inc(x_1); +x_44 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__7(x_1, x_41, 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 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastNeg___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__16(x_1, x_45, x_46); +x_48 = lean_ctor_get(x_47, 0); +lean_inc(x_48); +x_49 = lean_ctor_get(x_47, 1); +lean_inc(x_49); +lean_dec(x_47); +lean_inc(x_8); +lean_inc(x_11); +x_50 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_50, 0, x_11); +lean_ctor_set(x_50, 1, x_8); +lean_inc(x_1); +x_51 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__7(x_1, x_48, x_50); +x_52 = lean_ctor_get(x_51, 0); +lean_inc(x_52); +x_53 = lean_ctor_get(x_51, 1); +lean_inc(x_53); +lean_dec(x_51); +x_54 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastNeg___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__16(x_1, x_52, 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_alloc_ctor(0, 2, 0); +lean_ctor_set(x_57, 0, x_11); +lean_ctor_set(x_57, 1, x_39); +lean_inc(x_1); +x_58 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__7(x_1, x_55, 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); +lean_inc(x_1); +x_61 = lean_alloc_ctor(0, 7, 0); +lean_ctor_set(x_61, 0, x_1); +lean_ctor_set(x_61, 1, x_7); +lean_ctor_set(x_61, 2, x_8); +lean_ctor_set(x_61, 3, x_42); +lean_ctor_set(x_61, 4, x_49); +lean_ctor_set(x_61, 5, x_56); +lean_ctor_set(x_61, 6, x_60); +x_62 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv_signBranch___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__25(x_1, x_59, x_61); +lean_dec(x_61); +lean_dec(x_1); +return x_62; +} +} +else +{ +lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; +x_63 = lean_ctor_get(x_3, 0); +x_64 = lean_ctor_get(x_3, 1); +lean_inc(x_64); +lean_inc(x_63); +lean_dec(x_3); +lean_inc(x_63); +x_65 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastNeg___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__16(x_1, x_2, x_63); +x_66 = lean_ctor_get(x_65, 0); +lean_inc(x_66); +x_67 = lean_ctor_get(x_65, 1); +lean_inc(x_67); +lean_dec(x_65); +lean_inc(x_64); +x_68 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastNeg___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__16(x_1, x_66, x_64); +x_69 = lean_ctor_get(x_68, 0); +lean_inc(x_69); +x_70 = lean_ctor_get(x_68, 1); +lean_inc(x_70); +if (lean_is_exclusive(x_68)) { + lean_ctor_release(x_68, 0); + lean_ctor_release(x_68, 1); + x_71 = x_68; +} else { + lean_dec_ref(x_68); + x_71 = lean_box(0); +} +lean_inc(x_64); +lean_inc(x_63); +x_72 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_72, 0, x_63); +lean_ctor_set(x_72, 1, x_64); +lean_inc(x_1); +x_73 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__7(x_1, x_69, x_72); +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_inc(x_70); +lean_inc(x_63); +if (lean_is_scalar(x_71)) { + x_76 = lean_alloc_ctor(0, 2, 0); +} else { + x_76 = x_71; +} +lean_ctor_set(x_76, 0, x_63); +lean_ctor_set(x_76, 1, x_70); +lean_inc(x_1); +x_77 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__7(x_1, x_74, x_76); +x_78 = lean_ctor_get(x_77, 0); +lean_inc(x_78); +x_79 = lean_ctor_get(x_77, 1); +lean_inc(x_79); +lean_dec(x_77); +x_80 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastNeg___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__16(x_1, x_78, x_79); +x_81 = lean_ctor_get(x_80, 0); +lean_inc(x_81); +x_82 = lean_ctor_get(x_80, 1); +lean_inc(x_82); +lean_dec(x_80); +lean_inc(x_64); +lean_inc(x_67); +x_83 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_83, 0, x_67); +lean_ctor_set(x_83, 1, x_64); +lean_inc(x_1); +x_84 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__7(x_1, x_81, x_83); +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_Std_Tactic_BVDecide_BVExpr_bitblast_blastNeg___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__16(x_1, x_85, x_86); +x_88 = lean_ctor_get(x_87, 0); +lean_inc(x_88); +x_89 = lean_ctor_get(x_87, 1); +lean_inc(x_89); +lean_dec(x_87); +x_90 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_90, 0, x_67); +lean_ctor_set(x_90, 1, x_70); +lean_inc(x_1); +x_91 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__7(x_1, x_88, x_90); +x_92 = lean_ctor_get(x_91, 0); +lean_inc(x_92); +x_93 = lean_ctor_get(x_91, 1); +lean_inc(x_93); +lean_dec(x_91); +lean_inc(x_1); +x_94 = lean_alloc_ctor(0, 7, 0); +lean_ctor_set(x_94, 0, x_1); +lean_ctor_set(x_94, 1, x_63); +lean_ctor_set(x_94, 2, x_64); +lean_ctor_set(x_94, 3, x_75); +lean_ctor_set(x_94, 4, x_82); +lean_ctor_set(x_94, 5, x_89); +lean_ctor_set(x_94, 6, x_93); +x_95 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv_signBranch___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__25(x_1, x_92, x_94); +lean_dec(x_94); +lean_dec(x_1); +return x_95; +} +} +else +{ +lean_object* x_96; lean_object* x_97; +lean_dec(x_3); +lean_dec(x_1); +x_96 = l_Std_Sat_AIG_RefVec_empty___at_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul_go___spec__2(x_2); +x_97 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_97, 0, x_2); +lean_ctor_set(x_97, 1, x_96); +return x_97; +} +} +} +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRightConst_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__27(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { uint8_t x_8; @@ -1523,7 +1869,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRightConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__24(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRightConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__26(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; @@ -1531,11 +1877,11 @@ x_4 = lean_ctor_get(x_3, 0); x_5 = lean_ctor_get(x_3, 1); x_6 = l_Std_Sat_AIG_RefVec_empty___at_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul_go___spec__2(x_2); x_7 = lean_unsigned_to_nat(0u); -x_8 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRightConst_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__25(x_1, x_2, x_4, x_5, x_7, lean_box(0), x_6); +x_8 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRightConst_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__27(x_1, x_2, x_4, x_5, x_7, lean_box(0), x_6); return x_8; } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateLeft_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__27(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateLeft_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__29(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { uint8_t x_8; @@ -1587,7 +1933,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateLeft___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__26(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateLeft___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__28(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -1599,7 +1945,7 @@ x_5 = lean_ctor_get(x_3, 0); x_6 = lean_ctor_get(x_3, 1); x_7 = l_Std_Sat_AIG_RefVec_empty___at_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul_go___spec__2(x_2); x_8 = lean_unsigned_to_nat(0u); -x_9 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateLeft_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__27(x_1, x_2, x_5, x_6, x_8, lean_box(0), x_7); +x_9 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateLeft_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__29(x_1, x_2, x_5, x_6, x_8, lean_box(0), x_7); lean_dec(x_6); lean_dec(x_5); lean_ctor_set(x_3, 1, x_9); @@ -1616,7 +1962,7 @@ lean_inc(x_10); lean_dec(x_3); x_12 = l_Std_Sat_AIG_RefVec_empty___at_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul_go___spec__2(x_2); x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateLeft_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__27(x_1, x_2, x_10, x_11, x_13, lean_box(0), x_12); +x_14 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateLeft_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__29(x_1, x_2, x_10, x_11, x_13, lean_box(0), x_12); lean_dec(x_11); lean_dec(x_10); x_15 = lean_alloc_ctor(0, 2, 0); @@ -1626,7 +1972,7 @@ return x_15; } } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateRight_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__29(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateRight_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__31(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { uint8_t x_8; @@ -1679,7 +2025,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateRight___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__28(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateRight___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__30(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -1691,7 +2037,7 @@ x_5 = lean_ctor_get(x_3, 0); x_6 = lean_ctor_get(x_3, 1); x_7 = l_Std_Sat_AIG_RefVec_empty___at_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul_go___spec__2(x_2); x_8 = lean_unsigned_to_nat(0u); -x_9 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateRight_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__29(x_1, x_2, x_5, x_6, x_8, lean_box(0), x_7); +x_9 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateRight_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__31(x_1, x_2, x_5, x_6, x_8, lean_box(0), x_7); lean_dec(x_6); lean_dec(x_5); lean_ctor_set(x_3, 1, x_9); @@ -1708,7 +2054,7 @@ lean_inc(x_10); lean_dec(x_3); x_12 = l_Std_Sat_AIG_RefVec_empty___at_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul_go___spec__2(x_2); x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateRight_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__29(x_1, x_2, x_10, x_11, x_13, lean_box(0), x_12); +x_14 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateRight_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__31(x_1, x_2, x_10, x_11, x_13, lean_box(0), x_12); lean_dec(x_11); lean_dec(x_10); x_15 = lean_alloc_ctor(0, 2, 0); @@ -1718,7 +2064,7 @@ return x_15; } } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastArithShiftRightConst_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__31(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastArithShiftRightConst_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__33(lean_object* x_1, 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; @@ -1766,7 +2112,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastArithShiftRightConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__30(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastArithShiftRightConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__32(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -1778,7 +2124,7 @@ x_5 = lean_ctor_get(x_3, 0); x_6 = lean_ctor_get(x_3, 1); x_7 = l_Std_Sat_AIG_RefVec_empty___at_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul_go___spec__2(x_2); x_8 = lean_unsigned_to_nat(0u); -x_9 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastArithShiftRightConst_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__31(x_1, x_2, x_5, x_6, x_8, lean_box(0), x_7); +x_9 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastArithShiftRightConst_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__33(x_1, x_2, x_5, x_6, x_8, lean_box(0), x_7); lean_dec(x_6); lean_dec(x_5); lean_ctor_set(x_3, 1, x_9); @@ -1795,7 +2141,7 @@ lean_inc(x_10); lean_dec(x_3); x_12 = l_Std_Sat_AIG_RefVec_empty___at_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul_go___spec__2(x_2); x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastArithShiftRightConst_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__31(x_1, x_2, x_10, x_11, x_13, lean_box(0), x_12); +x_14 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastArithShiftRightConst_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__33(x_1, x_2, x_10, x_11, x_13, lean_box(0), x_12); lean_dec(x_11); lean_dec(x_10); x_15 = lean_alloc_ctor(0, 2, 0); @@ -1805,7 +2151,7 @@ return x_15; } } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastAppend___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__32(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastAppend___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__34(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; @@ -1822,7 +2168,7 @@ lean_ctor_set(x_7, 1, x_6); return x_7; } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastReplicate_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__34(lean_object* x_1, lean_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_Tactic_BVDecide_BVExpr_bitblast_blastReplicate_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__36(lean_object* x_1, 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; @@ -1846,7 +2192,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastReplicate___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__33(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastReplicate___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__35(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; @@ -1855,14 +2201,14 @@ x_5 = lean_ctor_get(x_3, 1); x_6 = lean_ctor_get(x_3, 2); x_7 = l_Std_Sat_AIG_RefVec_empty___at_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul_go___spec__2(x_2); x_8 = lean_unsigned_to_nat(0u); -x_9 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastReplicate_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__34(x_2, x_4, x_5, x_6, x_8, lean_box(0), x_7); +x_9 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastReplicate_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__36(x_2, x_4, x_5, x_6, x_8, lean_box(0), x_7); x_10 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_10, 0, x_2); lean_ctor_set(x_10, 1, x_9); return x_10; } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSignExtend_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__36(lean_object* x_1, lean_object* x_2, lean_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_Std_Tactic_BVDecide_BVExpr_bitblast_blastSignExtend_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__38(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { uint8_t x_9; @@ -1909,7 +2255,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSignExtend___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__35(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSignExtend___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__37(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -1926,7 +2272,7 @@ if (x_8 == 0) lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_free_object(x_3); x_9 = l_Std_Sat_AIG_RefVec_empty___at_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul_go___spec__2(x_2); -x_10 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSignExtend_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__36(x_2, x_5, lean_box(0), x_6, x_1, x_7, lean_box(0), x_9); +x_10 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSignExtend_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__38(x_2, x_5, lean_box(0), x_6, x_1, x_7, lean_box(0), x_9); lean_dec(x_6); lean_dec(x_5); x_11 = lean_alloc_ctor(0, 2, 0); @@ -1956,7 +2302,7 @@ if (x_16 == 0) { lean_object* x_17; lean_object* x_18; lean_object* x_19; x_17 = l_Std_Sat_AIG_RefVec_empty___at_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul_go___spec__2(x_2); -x_18 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSignExtend_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__36(x_2, x_13, lean_box(0), x_14, x_1, x_15, lean_box(0), x_17); +x_18 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSignExtend_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__38(x_2, x_13, lean_box(0), x_14, x_1, x_15, lean_box(0), x_17); lean_dec(x_14); lean_dec(x_13); x_19 = lean_alloc_ctor(0, 2, 0); @@ -1977,7 +2323,7 @@ return x_21; } } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft_twoPowShift___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__38(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft_twoPowShift___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__40(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; uint8_t x_8; @@ -2022,7 +2368,7 @@ return x_18; } } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___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) { +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___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) { _start: { lean_object* x_7; lean_object* x_8; uint8_t x_9; @@ -2054,7 +2400,7 @@ lean_ctor_set(x_12, 0, x_2); lean_ctor_set(x_12, 1, x_6); lean_ctor_set(x_12, 2, x_4); lean_ctor_set(x_12, 3, x_11); -x_13 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft_twoPowShift___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__38(x_1, x_3, x_12); +x_13 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft_twoPowShift___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__40(x_1, x_3, x_12); lean_dec(x_12); x_14 = lean_ctor_get(x_13, 0); lean_inc(x_14); @@ -2068,7 +2414,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__37(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__39(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; uint8_t x_8; @@ -2091,14 +2437,14 @@ lean_ctor_set(x_9, 0, x_4); lean_ctor_set(x_9, 1, x_5); lean_ctor_set(x_9, 2, x_6); lean_ctor_set(x_9, 3, x_7); -x_10 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft_twoPowShift___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__38(x_1, x_2, x_9); +x_10 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft_twoPowShift___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__40(x_1, x_2, x_9); lean_dec(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_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__39(x_1, x_4, x_11, x_6, x_7, x_12); +x_13 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__41(x_1, x_4, x_11, x_6, x_7, x_12); return x_13; } else @@ -2113,7 +2459,7 @@ return x_14; } } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight_twoPowShift___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__41(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight_twoPowShift___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__43(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; uint8_t x_8; @@ -2140,7 +2486,7 @@ lean_inc(x_5); x_12 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_12, 0, x_5); lean_ctor_set(x_12, 1, x_11); -x_13 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRightConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__24(x_1, x_2, x_12); +x_13 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRightConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__26(x_1, x_2, x_12); lean_dec(x_12); x_14 = lean_ctor_get(x_13, 0); lean_inc(x_14); @@ -2158,7 +2504,7 @@ return x_18; } } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__42(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__44(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; lean_object* x_8; uint8_t x_9; @@ -2190,7 +2536,7 @@ lean_ctor_set(x_12, 0, x_2); lean_ctor_set(x_12, 1, x_6); lean_ctor_set(x_12, 2, x_4); lean_ctor_set(x_12, 3, x_11); -x_13 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight_twoPowShift___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__41(x_1, x_3, x_12); +x_13 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight_twoPowShift___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__43(x_1, x_3, x_12); lean_dec(x_12); x_14 = lean_ctor_get(x_13, 0); lean_inc(x_14); @@ -2204,7 +2550,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__40(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__42(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; uint8_t x_8; @@ -2227,14 +2573,14 @@ lean_ctor_set(x_9, 0, x_4); lean_ctor_set(x_9, 1, x_5); lean_ctor_set(x_9, 2, x_6); lean_ctor_set(x_9, 3, x_7); -x_10 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight_twoPowShift___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__41(x_1, x_2, x_9); +x_10 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight_twoPowShift___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__43(x_1, x_2, x_9); lean_dec(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_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__42(x_1, x_4, x_11, x_6, x_7, x_12); +x_13 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__44(x_1, x_4, x_11, x_6, x_7, x_12); return x_13; } else @@ -2568,7 +2914,7 @@ x_81 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv___at_Std_Tactic_BVDecide_ return x_81; } } -default: +case 6: { uint8_t x_82; lean_free_object(x_29); @@ -2596,62 +2942,60 @@ x_88 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUmod___at_Std_Tactic_BVDecide_ return x_88; } } +default: +{ +uint8_t x_89; +lean_free_object(x_29); +x_89 = !lean_is_exclusive(x_33); +if (x_89 == 0) +{ +lean_object* x_90; lean_object* x_91; +x_90 = lean_ctor_get(x_33, 0); +lean_ctor_set(x_33, 0, x_32); +x_91 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__24(x_1, x_90, x_33); +return x_91; +} +else +{ +lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; +x_92 = lean_ctor_get(x_33, 0); +x_93 = lean_ctor_get(x_33, 1); +lean_inc(x_93); +lean_inc(x_92); +lean_dec(x_33); +x_94 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_94, 0, x_32); +lean_ctor_set(x_94, 1, x_93); +x_95 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__24(x_1, x_92, x_94); +return x_95; +} +} } } else { -lean_object* x_89; lean_object* x_90; lean_object* x_91; -x_89 = lean_ctor_get(x_29, 0); -x_90 = lean_ctor_get(x_29, 1); -lean_inc(x_90); -lean_inc(x_89); +lean_object* x_96; lean_object* x_97; lean_object* x_98; +x_96 = lean_ctor_get(x_29, 0); +x_97 = lean_ctor_get(x_29, 1); +lean_inc(x_97); +lean_inc(x_96); lean_dec(x_29); lean_inc(x_1); -x_91 = l_Std_Tactic_BVDecide_BVExpr_bitblast_go(x_1, x_89, x_28); +x_98 = l_Std_Tactic_BVDecide_BVExpr_bitblast_go(x_1, x_96, x_28); switch (x_27) { case 0: { -lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; -x_92 = lean_ctor_get(x_91, 0); -lean_inc(x_92); -x_93 = lean_ctor_get(x_91, 1); -lean_inc(x_93); -if (lean_is_exclusive(x_91)) { - lean_ctor_release(x_91, 0); - lean_ctor_release(x_91, 1); - x_94 = x_91; -} else { - lean_dec_ref(x_91); - x_94 = lean_box(0); -} -if (lean_is_scalar(x_94)) { - x_95 = lean_alloc_ctor(0, 2, 0); -} else { - x_95 = x_94; -} -lean_ctor_set(x_95, 0, x_90); -lean_ctor_set(x_95, 1, x_93); -x_96 = l_Std_Tactic_BVDecide_BVPred_mkEq___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__8___closed__2; -x_97 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_97, 0, x_95); -lean_ctor_set(x_97, 1, x_96); -x_98 = l_Std_Sat_AIG_RefVec_zip___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__5(x_1, x_92, x_97); -lean_dec(x_1); -return x_98; -} -case 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; -x_99 = lean_ctor_get(x_91, 0); +x_99 = lean_ctor_get(x_98, 0); lean_inc(x_99); -x_100 = lean_ctor_get(x_91, 1); +x_100 = lean_ctor_get(x_98, 1); lean_inc(x_100); -if (lean_is_exclusive(x_91)) { - lean_ctor_release(x_91, 0); - lean_ctor_release(x_91, 1); - x_101 = x_91; +if (lean_is_exclusive(x_98)) { + lean_ctor_release(x_98, 0); + lean_ctor_release(x_98, 1); + x_101 = x_98; } else { - lean_dec_ref(x_91); + lean_dec_ref(x_98); x_101 = lean_box(0); } if (lean_is_scalar(x_101)) { @@ -2659,9 +3003,9 @@ if (lean_is_scalar(x_101)) { } else { x_102 = x_101; } -lean_ctor_set(x_102, 0, x_90); +lean_ctor_set(x_102, 0, x_97); lean_ctor_set(x_102, 1, x_100); -x_103 = l_Std_Tactic_BVDecide_BVExpr_bitblast_go___closed__1; +x_103 = l_Std_Tactic_BVDecide_BVPred_mkEq___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__8___closed__2; x_104 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_104, 0, x_102); lean_ctor_set(x_104, 1, x_103); @@ -2669,19 +3013,19 @@ x_105 = l_Std_Sat_AIG_RefVec_zip___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___s lean_dec(x_1); return x_105; } -case 2: +case 1: { 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_106 = lean_ctor_get(x_91, 0); +x_106 = lean_ctor_get(x_98, 0); lean_inc(x_106); -x_107 = lean_ctor_get(x_91, 1); +x_107 = lean_ctor_get(x_98, 1); lean_inc(x_107); -if (lean_is_exclusive(x_91)) { - lean_ctor_release(x_91, 0); - lean_ctor_release(x_91, 1); - x_108 = x_91; +if (lean_is_exclusive(x_98)) { + lean_ctor_release(x_98, 0); + lean_ctor_release(x_98, 1); + x_108 = x_98; } else { - lean_dec_ref(x_91); + lean_dec_ref(x_98); x_108 = lean_box(0); } if (lean_is_scalar(x_108)) { @@ -2689,9 +3033,9 @@ if (lean_is_scalar(x_108)) { } else { x_109 = x_108; } -lean_ctor_set(x_109, 0, x_90); +lean_ctor_set(x_109, 0, x_97); lean_ctor_set(x_109, 1, x_107); -x_110 = l_Std_Tactic_BVDecide_BVExpr_bitblast_go___closed__2; +x_110 = l_Std_Tactic_BVDecide_BVExpr_bitblast_go___closed__1; x_111 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_111, 0, x_109); lean_ctor_set(x_111, 1, x_110); @@ -2699,19 +3043,19 @@ x_112 = l_Std_Sat_AIG_RefVec_zip___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___s lean_dec(x_1); return x_112; } -case 3: +case 2: { -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_91, 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; +x_113 = lean_ctor_get(x_98, 0); lean_inc(x_113); -x_114 = lean_ctor_get(x_91, 1); +x_114 = lean_ctor_get(x_98, 1); lean_inc(x_114); -if (lean_is_exclusive(x_91)) { - lean_ctor_release(x_91, 0); - lean_ctor_release(x_91, 1); - x_115 = x_91; +if (lean_is_exclusive(x_98)) { + lean_ctor_release(x_98, 0); + lean_ctor_release(x_98, 1); + x_115 = x_98; } else { - lean_dec_ref(x_91); + lean_dec_ref(x_98); x_115 = lean_box(0); } if (lean_is_scalar(x_115)) { @@ -2719,352 +3063,373 @@ if (lean_is_scalar(x_115)) { } else { x_116 = x_115; } -lean_ctor_set(x_116, 0, x_90); +lean_ctor_set(x_116, 0, x_97); lean_ctor_set(x_116, 1, x_114); -x_117 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastAdd___at_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul_go___spec__16(x_1, x_113, x_116); -lean_dec(x_116); +x_117 = l_Std_Tactic_BVDecide_BVExpr_bitblast_go___closed__2; +x_118 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_118, 0, x_116); +lean_ctor_set(x_118, 1, x_117); +x_119 = l_Std_Sat_AIG_RefVec_zip___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__5(x_1, x_113, x_118); +lean_dec(x_1); +return x_119; +} +case 3: +{ +lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; +x_120 = lean_ctor_get(x_98, 0); +lean_inc(x_120); +x_121 = lean_ctor_get(x_98, 1); +lean_inc(x_121); +if (lean_is_exclusive(x_98)) { + lean_ctor_release(x_98, 0); + lean_ctor_release(x_98, 1); + x_122 = x_98; +} else { + lean_dec_ref(x_98); + x_122 = lean_box(0); +} +if (lean_is_scalar(x_122)) { + x_123 = lean_alloc_ctor(0, 2, 0); +} else { + x_123 = x_122; +} +lean_ctor_set(x_123, 0, x_97); +lean_ctor_set(x_123, 1, x_121); +x_124 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastAdd___at_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul_go___spec__16(x_1, x_120, x_123); +lean_dec(x_123); lean_dec(x_1); -return x_117; +return x_124; } case 4: { -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_91, 0); -lean_inc(x_118); -x_119 = lean_ctor_get(x_91, 1); -lean_inc(x_119); -if (lean_is_exclusive(x_91)) { - lean_ctor_release(x_91, 0); - lean_ctor_release(x_91, 1); - x_120 = x_91; +lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; +x_125 = lean_ctor_get(x_98, 0); +lean_inc(x_125); +x_126 = lean_ctor_get(x_98, 1); +lean_inc(x_126); +if (lean_is_exclusive(x_98)) { + lean_ctor_release(x_98, 0); + lean_ctor_release(x_98, 1); + x_127 = x_98; } else { - lean_dec_ref(x_91); - x_120 = lean_box(0); + lean_dec_ref(x_98); + x_127 = lean_box(0); } -if (lean_is_scalar(x_120)) { - x_121 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_127)) { + x_128 = lean_alloc_ctor(0, 2, 0); } else { - x_121 = x_120; + x_128 = x_127; } -lean_ctor_set(x_121, 0, x_90); -lean_ctor_set(x_121, 1, x_119); -x_122 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul(x_1, x_118, x_121); +lean_ctor_set(x_128, 0, x_97); +lean_ctor_set(x_128, 1, x_126); +x_129 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul(x_1, x_125, x_128); lean_dec(x_1); -return x_122; +return x_129; } case 5: { -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_91, 0); -lean_inc(x_123); -x_124 = lean_ctor_get(x_91, 1); -lean_inc(x_124); -if (lean_is_exclusive(x_91)) { - lean_ctor_release(x_91, 0); - lean_ctor_release(x_91, 1); - x_125 = x_91; +lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; +x_130 = lean_ctor_get(x_98, 0); +lean_inc(x_130); +x_131 = lean_ctor_get(x_98, 1); +lean_inc(x_131); +if (lean_is_exclusive(x_98)) { + lean_ctor_release(x_98, 0); + lean_ctor_release(x_98, 1); + x_132 = x_98; +} else { + lean_dec_ref(x_98); + x_132 = lean_box(0); +} +if (lean_is_scalar(x_132)) { + x_133 = lean_alloc_ctor(0, 2, 0); +} else { + x_133 = x_132; +} +lean_ctor_set(x_133, 0, x_97); +lean_ctor_set(x_133, 1, x_131); +x_134 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__7(x_1, x_130, x_133); +return x_134; +} +case 6: +{ +lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; +x_135 = lean_ctor_get(x_98, 0); +lean_inc(x_135); +x_136 = lean_ctor_get(x_98, 1); +lean_inc(x_136); +if (lean_is_exclusive(x_98)) { + lean_ctor_release(x_98, 0); + lean_ctor_release(x_98, 1); + x_137 = x_98; } else { - lean_dec_ref(x_91); - x_125 = lean_box(0); + lean_dec_ref(x_98); + x_137 = lean_box(0); } -if (lean_is_scalar(x_125)) { - x_126 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_137)) { + x_138 = lean_alloc_ctor(0, 2, 0); } else { - x_126 = x_125; + x_138 = x_137; } -lean_ctor_set(x_126, 0, x_90); -lean_ctor_set(x_126, 1, x_124); -x_127 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__7(x_1, x_123, x_126); -return x_127; +lean_ctor_set(x_138, 0, x_97); +lean_ctor_set(x_138, 1, x_136); +x_139 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUmod___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__23(x_1, x_135, x_138); +return x_139; } default: { -lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; -x_128 = lean_ctor_get(x_91, 0); -lean_inc(x_128); -x_129 = lean_ctor_get(x_91, 1); -lean_inc(x_129); -if (lean_is_exclusive(x_91)) { - lean_ctor_release(x_91, 0); - lean_ctor_release(x_91, 1); - x_130 = x_91; +lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; +x_140 = lean_ctor_get(x_98, 0); +lean_inc(x_140); +x_141 = lean_ctor_get(x_98, 1); +lean_inc(x_141); +if (lean_is_exclusive(x_98)) { + lean_ctor_release(x_98, 0); + lean_ctor_release(x_98, 1); + x_142 = x_98; } else { - lean_dec_ref(x_91); - x_130 = lean_box(0); + lean_dec_ref(x_98); + x_142 = lean_box(0); } -if (lean_is_scalar(x_130)) { - x_131 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_142)) { + x_143 = lean_alloc_ctor(0, 2, 0); } else { - x_131 = x_130; + x_143 = x_142; } -lean_ctor_set(x_131, 0, x_90); -lean_ctor_set(x_131, 1, x_129); -x_132 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUmod___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__23(x_1, x_128, x_131); -return x_132; +lean_ctor_set(x_143, 0, x_97); +lean_ctor_set(x_143, 1, x_141); +x_144 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__24(x_1, x_140, x_143); +return x_144; } } } } case 5: { -lean_object* x_133; lean_object* x_134; lean_object* x_135; -x_133 = lean_ctor_get(x_3, 1); -lean_inc(x_133); -x_134 = lean_ctor_get(x_3, 2); -lean_inc(x_134); +lean_object* x_145; lean_object* x_146; lean_object* x_147; +x_145 = lean_ctor_get(x_3, 1); +lean_inc(x_145); +x_146 = lean_ctor_get(x_3, 2); +lean_inc(x_146); lean_dec(x_3); lean_inc(x_1); -x_135 = l_Std_Tactic_BVDecide_BVExpr_bitblast_go(x_1, x_2, x_134); -switch (lean_obj_tag(x_133)) { +x_147 = l_Std_Tactic_BVDecide_BVExpr_bitblast_go(x_1, x_2, x_146); +switch (lean_obj_tag(x_145)) { case 0: { -lean_object* x_136; lean_object* x_137; lean_object* x_138; -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 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastNot___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__17(x_1, x_136, x_137); +lean_object* x_148; lean_object* x_149; lean_object* x_150; +x_148 = lean_ctor_get(x_147, 0); +lean_inc(x_148); +x_149 = lean_ctor_get(x_147, 1); +lean_inc(x_149); +lean_dec(x_147); +x_150 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastNot___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__17(x_1, x_148, x_149); lean_dec(x_1); -return x_138; +return x_150; } case 1: { -uint8_t x_139; -x_139 = !lean_is_exclusive(x_135); -if (x_139 == 0) +uint8_t x_151; +x_151 = !lean_is_exclusive(x_147); +if (x_151 == 0) { -lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; -x_140 = lean_ctor_get(x_135, 0); -x_141 = lean_ctor_get(x_135, 1); -x_142 = lean_ctor_get(x_133, 0); -lean_inc(x_142); -lean_dec(x_133); -lean_ctor_set(x_135, 1, x_142); -lean_ctor_set(x_135, 0, x_141); -x_143 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeftConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul_go___spec__1(x_1, x_140, x_135); -lean_dec(x_135); +lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; +x_152 = lean_ctor_get(x_147, 0); +x_153 = lean_ctor_get(x_147, 1); +x_154 = lean_ctor_get(x_145, 0); +lean_inc(x_154); +lean_dec(x_145); +lean_ctor_set(x_147, 1, x_154); +lean_ctor_set(x_147, 0, x_153); +x_155 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeftConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul_go___spec__1(x_1, x_152, x_147); +lean_dec(x_147); lean_dec(x_1); -return x_143; +return x_155; } else { -lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; -x_144 = lean_ctor_get(x_135, 0); -x_145 = lean_ctor_get(x_135, 1); -lean_inc(x_145); -lean_inc(x_144); -lean_dec(x_135); -x_146 = lean_ctor_get(x_133, 0); -lean_inc(x_146); -lean_dec(x_133); -x_147 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_147, 0, x_145); -lean_ctor_set(x_147, 1, x_146); -x_148 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeftConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul_go___spec__1(x_1, x_144, x_147); +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_147, 0); +x_157 = lean_ctor_get(x_147, 1); +lean_inc(x_157); +lean_inc(x_156); lean_dec(x_147); +x_158 = lean_ctor_get(x_145, 0); +lean_inc(x_158); +lean_dec(x_145); +x_159 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_159, 0, x_157); +lean_ctor_set(x_159, 1, x_158); +x_160 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeftConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_blastMul_go___spec__1(x_1, x_156, x_159); +lean_dec(x_159); lean_dec(x_1); -return x_148; +return x_160; } } case 2: { -uint8_t x_149; -x_149 = !lean_is_exclusive(x_135); -if (x_149 == 0) +uint8_t x_161; +x_161 = !lean_is_exclusive(x_147); +if (x_161 == 0) { -lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; -x_150 = lean_ctor_get(x_135, 0); -x_151 = lean_ctor_get(x_135, 1); -x_152 = lean_ctor_get(x_133, 0); -lean_inc(x_152); -lean_dec(x_133); -lean_ctor_set(x_135, 1, x_152); -lean_ctor_set(x_135, 0, x_151); -x_153 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRightConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__24(x_1, x_150, x_135); -lean_dec(x_135); +lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; +x_162 = lean_ctor_get(x_147, 0); +x_163 = lean_ctor_get(x_147, 1); +x_164 = lean_ctor_get(x_145, 0); +lean_inc(x_164); +lean_dec(x_145); +lean_ctor_set(x_147, 1, x_164); +lean_ctor_set(x_147, 0, x_163); +x_165 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRightConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__26(x_1, x_162, x_147); +lean_dec(x_147); lean_dec(x_1); -return x_153; +return x_165; } else { -lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; -x_154 = lean_ctor_get(x_135, 0); -x_155 = lean_ctor_get(x_135, 1); -lean_inc(x_155); -lean_inc(x_154); -lean_dec(x_135); -x_156 = lean_ctor_get(x_133, 0); -lean_inc(x_156); -lean_dec(x_133); -x_157 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_157, 0, x_155); -lean_ctor_set(x_157, 1, x_156); -x_158 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRightConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__24(x_1, x_154, x_157); -lean_dec(x_157); +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_147, 0); +x_167 = lean_ctor_get(x_147, 1); +lean_inc(x_167); +lean_inc(x_166); +lean_dec(x_147); +x_168 = lean_ctor_get(x_145, 0); +lean_inc(x_168); +lean_dec(x_145); +x_169 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_169, 0, x_167); +lean_ctor_set(x_169, 1, x_168); +x_170 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRightConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__26(x_1, x_166, x_169); +lean_dec(x_169); lean_dec(x_1); -return x_158; +return x_170; } } case 3: { -uint8_t x_159; -x_159 = !lean_is_exclusive(x_135); -if (x_159 == 0) +uint8_t x_171; +x_171 = !lean_is_exclusive(x_147); +if (x_171 == 0) { -lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; -x_160 = lean_ctor_get(x_135, 0); -x_161 = lean_ctor_get(x_135, 1); -x_162 = lean_ctor_get(x_133, 0); -lean_inc(x_162); -lean_dec(x_133); -lean_ctor_set(x_135, 1, x_162); -lean_ctor_set(x_135, 0, x_161); -x_163 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateLeft___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__26(x_1, x_160, x_135); +lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; +x_172 = lean_ctor_get(x_147, 0); +x_173 = lean_ctor_get(x_147, 1); +x_174 = lean_ctor_get(x_145, 0); +lean_inc(x_174); +lean_dec(x_145); +lean_ctor_set(x_147, 1, x_174); +lean_ctor_set(x_147, 0, x_173); +x_175 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateLeft___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__28(x_1, x_172, x_147); lean_dec(x_1); -return x_163; +return x_175; } else { -lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; -x_164 = lean_ctor_get(x_135, 0); -x_165 = lean_ctor_get(x_135, 1); -lean_inc(x_165); -lean_inc(x_164); -lean_dec(x_135); -x_166 = lean_ctor_get(x_133, 0); -lean_inc(x_166); -lean_dec(x_133); -x_167 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_167, 0, x_165); -lean_ctor_set(x_167, 1, x_166); -x_168 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateLeft___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__26(x_1, x_164, x_167); +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_147, 0); +x_177 = lean_ctor_get(x_147, 1); +lean_inc(x_177); +lean_inc(x_176); +lean_dec(x_147); +x_178 = lean_ctor_get(x_145, 0); +lean_inc(x_178); +lean_dec(x_145); +x_179 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_179, 0, x_177); +lean_ctor_set(x_179, 1, x_178); +x_180 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateLeft___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__28(x_1, x_176, x_179); lean_dec(x_1); -return x_168; +return x_180; } } case 4: { -uint8_t x_169; -x_169 = !lean_is_exclusive(x_135); -if (x_169 == 0) +uint8_t x_181; +x_181 = !lean_is_exclusive(x_147); +if (x_181 == 0) { -lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; -x_170 = lean_ctor_get(x_135, 0); -x_171 = lean_ctor_get(x_135, 1); -x_172 = lean_ctor_get(x_133, 0); -lean_inc(x_172); -lean_dec(x_133); -lean_ctor_set(x_135, 1, x_172); -lean_ctor_set(x_135, 0, x_171); -x_173 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateRight___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__28(x_1, x_170, x_135); +lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; +x_182 = lean_ctor_get(x_147, 0); +x_183 = lean_ctor_get(x_147, 1); +x_184 = lean_ctor_get(x_145, 0); +lean_inc(x_184); +lean_dec(x_145); +lean_ctor_set(x_147, 1, x_184); +lean_ctor_set(x_147, 0, x_183); +x_185 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateRight___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__30(x_1, x_182, x_147); lean_dec(x_1); -return x_173; +return x_185; } 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_135, 0); -x_175 = lean_ctor_get(x_135, 1); -lean_inc(x_175); -lean_inc(x_174); -lean_dec(x_135); -x_176 = lean_ctor_get(x_133, 0); -lean_inc(x_176); -lean_dec(x_133); -x_177 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_177, 0, x_175); -lean_ctor_set(x_177, 1, x_176); -x_178 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateRight___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__28(x_1, x_174, x_177); +lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; +x_186 = lean_ctor_get(x_147, 0); +x_187 = lean_ctor_get(x_147, 1); +lean_inc(x_187); +lean_inc(x_186); +lean_dec(x_147); +x_188 = lean_ctor_get(x_145, 0); +lean_inc(x_188); +lean_dec(x_145); +x_189 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_189, 0, x_187); +lean_ctor_set(x_189, 1, x_188); +x_190 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateRight___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__30(x_1, x_186, x_189); lean_dec(x_1); -return x_178; +return x_190; } } default: { -uint8_t x_179; -x_179 = !lean_is_exclusive(x_135); -if (x_179 == 0) -{ -lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; -x_180 = lean_ctor_get(x_135, 0); -x_181 = lean_ctor_get(x_135, 1); -x_182 = lean_ctor_get(x_133, 0); -lean_inc(x_182); -lean_dec(x_133); -lean_ctor_set(x_135, 1, x_182); -lean_ctor_set(x_135, 0, x_181); -x_183 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastArithShiftRightConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__30(x_1, x_180, x_135); +uint8_t x_191; +x_191 = !lean_is_exclusive(x_147); +if (x_191 == 0) +{ +lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; +x_192 = lean_ctor_get(x_147, 0); +x_193 = lean_ctor_get(x_147, 1); +x_194 = lean_ctor_get(x_145, 0); +lean_inc(x_194); +lean_dec(x_145); +lean_ctor_set(x_147, 1, x_194); +lean_ctor_set(x_147, 0, x_193); +x_195 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastArithShiftRightConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__32(x_1, x_192, x_147); lean_dec(x_1); -return x_183; +return x_195; } else { -lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; -x_184 = lean_ctor_get(x_135, 0); -x_185 = lean_ctor_get(x_135, 1); -lean_inc(x_185); -lean_inc(x_184); -lean_dec(x_135); -x_186 = lean_ctor_get(x_133, 0); -lean_inc(x_186); -lean_dec(x_133); -x_187 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_187, 0, x_185); -lean_ctor_set(x_187, 1, x_186); -x_188 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastArithShiftRightConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__30(x_1, x_184, x_187); +lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; +x_196 = lean_ctor_get(x_147, 0); +x_197 = lean_ctor_get(x_147, 1); +lean_inc(x_197); +lean_inc(x_196); +lean_dec(x_147); +x_198 = lean_ctor_get(x_145, 0); +lean_inc(x_198); +lean_dec(x_145); +x_199 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_199, 0, x_197); +lean_ctor_set(x_199, 1, x_198); +x_200 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastArithShiftRightConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__32(x_1, x_196, x_199); lean_dec(x_1); -return x_188; +return x_200; } } } } case 6: { -uint8_t x_189; -lean_dec(x_1); -x_189 = !lean_is_exclusive(x_3); -if (x_189 == 0) -{ -lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; -x_190 = lean_ctor_get(x_3, 0); -x_191 = lean_ctor_get(x_3, 1); -x_192 = lean_ctor_get(x_3, 2); -x_193 = lean_ctor_get(x_3, 3); -lean_inc(x_190); -x_194 = l_Std_Tactic_BVDecide_BVExpr_bitblast_go(x_190, x_2, x_192); -x_195 = lean_ctor_get(x_194, 0); -lean_inc(x_195); -x_196 = lean_ctor_get(x_194, 1); -lean_inc(x_196); -lean_dec(x_194); -lean_inc(x_191); -x_197 = l_Std_Tactic_BVDecide_BVExpr_bitblast_go(x_191, x_195, x_193); -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_nat_add(x_190, x_191); -lean_ctor_set_tag(x_3, 0); -lean_ctor_set(x_3, 3, x_199); -lean_ctor_set(x_3, 2, x_196); -x_201 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastAppend___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__32(x_200, x_198, x_3); -lean_dec(x_200); -return x_201; -} -else +uint8_t x_201; +lean_dec(x_1); +x_201 = !lean_is_exclusive(x_3); +if (x_201 == 0) { -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_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_202 = lean_ctor_get(x_3, 0); x_203 = lean_ctor_get(x_3, 1); x_204 = lean_ctor_get(x_3, 2); x_205 = lean_ctor_get(x_3, 3); -lean_inc(x_205); -lean_inc(x_204); -lean_inc(x_203); -lean_inc(x_202); -lean_dec(x_3); lean_inc(x_202); x_206 = l_Std_Tactic_BVDecide_BVExpr_bitblast_go(x_202, x_2, x_204); x_207 = lean_ctor_get(x_206, 0); @@ -3080,169 +3445,203 @@ x_211 = lean_ctor_get(x_209, 1); lean_inc(x_211); lean_dec(x_209); x_212 = lean_nat_add(x_202, x_203); -x_213 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_213, 0, x_202); -lean_ctor_set(x_213, 1, x_203); -lean_ctor_set(x_213, 2, x_208); -lean_ctor_set(x_213, 3, x_211); -x_214 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastAppend___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__32(x_212, x_210, x_213); +lean_ctor_set_tag(x_3, 0); +lean_ctor_set(x_3, 3, x_211); +lean_ctor_set(x_3, 2, x_208); +x_213 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastAppend___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__34(x_212, x_210, x_3); lean_dec(x_212); -return x_214; +return x_213; +} +else +{ +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; +x_214 = lean_ctor_get(x_3, 0); +x_215 = lean_ctor_get(x_3, 1); +x_216 = lean_ctor_get(x_3, 2); +x_217 = lean_ctor_get(x_3, 3); +lean_inc(x_217); +lean_inc(x_216); +lean_inc(x_215); +lean_inc(x_214); +lean_dec(x_3); +lean_inc(x_214); +x_218 = l_Std_Tactic_BVDecide_BVExpr_bitblast_go(x_214, x_2, x_216); +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_215); +x_221 = l_Std_Tactic_BVDecide_BVExpr_bitblast_go(x_215, x_219, x_217); +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_nat_add(x_214, x_215); +x_225 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_225, 0, x_214); +lean_ctor_set(x_225, 1, x_215); +lean_ctor_set(x_225, 2, x_220); +lean_ctor_set(x_225, 3, x_223); +x_226 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastAppend___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__34(x_224, x_222, x_225); +lean_dec(x_224); +return x_226; } } case 7: { -uint8_t x_215; +uint8_t x_227; lean_dec(x_1); -x_215 = !lean_is_exclusive(x_3); -if (x_215 == 0) +x_227 = !lean_is_exclusive(x_3); +if (x_227 == 0) { -lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; -x_216 = lean_ctor_get(x_3, 0); -x_217 = lean_ctor_get(x_3, 1); -x_218 = lean_ctor_get(x_3, 2); -lean_inc(x_216); -x_219 = l_Std_Tactic_BVDecide_BVExpr_bitblast_go(x_216, x_2, 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_nat_mul(x_216, x_217); +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; +x_228 = lean_ctor_get(x_3, 0); +x_229 = lean_ctor_get(x_3, 1); +x_230 = lean_ctor_get(x_3, 2); +lean_inc(x_228); +x_231 = l_Std_Tactic_BVDecide_BVExpr_bitblast_go(x_228, x_2, x_230); +x_232 = lean_ctor_get(x_231, 0); +lean_inc(x_232); +x_233 = lean_ctor_get(x_231, 1); +lean_inc(x_233); +lean_dec(x_231); +x_234 = lean_nat_mul(x_228, x_229); lean_ctor_set_tag(x_3, 0); -lean_ctor_set(x_3, 2, x_221); -x_223 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastReplicate___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__33(x_222, x_220, x_3); +lean_ctor_set(x_3, 2, x_233); +x_235 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastReplicate___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__35(x_234, x_232, x_3); lean_dec(x_3); -lean_dec(x_222); -return x_223; +lean_dec(x_234); +return x_235; } else { -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; -x_224 = lean_ctor_get(x_3, 0); -x_225 = lean_ctor_get(x_3, 1); -x_226 = lean_ctor_get(x_3, 2); -lean_inc(x_226); -lean_inc(x_225); -lean_inc(x_224); +lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; +x_236 = lean_ctor_get(x_3, 0); +x_237 = lean_ctor_get(x_3, 1); +x_238 = lean_ctor_get(x_3, 2); +lean_inc(x_238); +lean_inc(x_237); +lean_inc(x_236); lean_dec(x_3); -lean_inc(x_224); -x_227 = l_Std_Tactic_BVDecide_BVExpr_bitblast_go(x_224, x_2, x_226); -x_228 = lean_ctor_get(x_227, 0); -lean_inc(x_228); -x_229 = lean_ctor_get(x_227, 1); -lean_inc(x_229); -lean_dec(x_227); -x_230 = lean_nat_mul(x_224, x_225); -x_231 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_231, 0, x_224); -lean_ctor_set(x_231, 1, x_225); -lean_ctor_set(x_231, 2, x_229); -x_232 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastReplicate___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__33(x_230, x_228, x_231); -lean_dec(x_231); -lean_dec(x_230); -return x_232; +lean_inc(x_236); +x_239 = l_Std_Tactic_BVDecide_BVExpr_bitblast_go(x_236, x_2, 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_nat_mul(x_236, x_237); +x_243 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_243, 0, x_236); +lean_ctor_set(x_243, 1, x_237); +lean_ctor_set(x_243, 2, x_241); +x_244 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastReplicate___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__35(x_242, x_240, x_243); +lean_dec(x_243); +lean_dec(x_242); +return x_244; } } case 8: { -lean_object* x_233; lean_object* x_234; lean_object* x_235; uint8_t x_236; -x_233 = lean_ctor_get(x_3, 0); -lean_inc(x_233); -x_234 = lean_ctor_get(x_3, 2); -lean_inc(x_234); +lean_object* x_245; lean_object* x_246; lean_object* x_247; uint8_t x_248; +x_245 = lean_ctor_get(x_3, 0); +lean_inc(x_245); +x_246 = lean_ctor_get(x_3, 2); +lean_inc(x_246); lean_dec(x_3); -lean_inc(x_233); -x_235 = l_Std_Tactic_BVDecide_BVExpr_bitblast_go(x_233, x_2, x_234); -x_236 = !lean_is_exclusive(x_235); -if (x_236 == 0) -{ -lean_object* x_237; lean_object* x_238; -x_237 = lean_ctor_get(x_235, 0); -lean_ctor_set(x_235, 0, x_233); -x_238 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSignExtend___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__35(x_1, x_237, x_235); +lean_inc(x_245); +x_247 = l_Std_Tactic_BVDecide_BVExpr_bitblast_go(x_245, x_2, x_246); +x_248 = !lean_is_exclusive(x_247); +if (x_248 == 0) +{ +lean_object* x_249; lean_object* x_250; +x_249 = lean_ctor_get(x_247, 0); +lean_ctor_set(x_247, 0, x_245); +x_250 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSignExtend___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__37(x_1, x_249, x_247); lean_dec(x_1); -return x_238; +return x_250; } else { -lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; -x_239 = lean_ctor_get(x_235, 0); -x_240 = lean_ctor_get(x_235, 1); -lean_inc(x_240); -lean_inc(x_239); -lean_dec(x_235); -x_241 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_241, 0, x_233); -lean_ctor_set(x_241, 1, x_240); -x_242 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSignExtend___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__35(x_1, x_239, x_241); +lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; +x_251 = lean_ctor_get(x_247, 0); +x_252 = lean_ctor_get(x_247, 1); +lean_inc(x_252); +lean_inc(x_251); +lean_dec(x_247); +x_253 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_253, 0, x_245); +lean_ctor_set(x_253, 1, x_252); +x_254 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSignExtend___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__37(x_1, x_251, x_253); lean_dec(x_1); -return x_242; +return x_254; } } case 9: { -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; -x_243 = lean_ctor_get(x_3, 1); -lean_inc(x_243); -x_244 = lean_ctor_get(x_3, 2); -lean_inc(x_244); -x_245 = lean_ctor_get(x_3, 3); -lean_inc(x_245); +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; +x_255 = lean_ctor_get(x_3, 1); +lean_inc(x_255); +x_256 = lean_ctor_get(x_3, 2); +lean_inc(x_256); +x_257 = lean_ctor_get(x_3, 3); +lean_inc(x_257); lean_dec(x_3); lean_inc(x_1); -x_246 = l_Std_Tactic_BVDecide_BVExpr_bitblast_go(x_1, x_2, x_244); -x_247 = lean_ctor_get(x_246, 0); -lean_inc(x_247); -x_248 = lean_ctor_get(x_246, 1); -lean_inc(x_248); -lean_dec(x_246); -lean_inc(x_243); -x_249 = l_Std_Tactic_BVDecide_BVExpr_bitblast_go(x_243, x_247, x_245); -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_alloc_ctor(0, 3, 0); -lean_ctor_set(x_252, 0, x_243); -lean_ctor_set(x_252, 1, x_248); -lean_ctor_set(x_252, 2, x_251); -x_253 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__37(x_1, x_250, x_252); +x_258 = l_Std_Tactic_BVDecide_BVExpr_bitblast_go(x_1, x_2, x_256); +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(x_255); +x_261 = l_Std_Tactic_BVDecide_BVExpr_bitblast_go(x_255, x_259, x_257); +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_alloc_ctor(0, 3, 0); +lean_ctor_set(x_264, 0, x_255); +lean_ctor_set(x_264, 1, x_260); +lean_ctor_set(x_264, 2, x_263); +x_265 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__39(x_1, x_262, x_264); lean_dec(x_1); -return x_253; +return x_265; } default: { -lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; -x_254 = lean_ctor_get(x_3, 1); -lean_inc(x_254); -x_255 = lean_ctor_get(x_3, 2); -lean_inc(x_255); -x_256 = lean_ctor_get(x_3, 3); -lean_inc(x_256); +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_266 = lean_ctor_get(x_3, 1); +lean_inc(x_266); +x_267 = lean_ctor_get(x_3, 2); +lean_inc(x_267); +x_268 = lean_ctor_get(x_3, 3); +lean_inc(x_268); lean_dec(x_3); lean_inc(x_1); -x_257 = l_Std_Tactic_BVDecide_BVExpr_bitblast_go(x_1, x_2, x_255); -x_258 = lean_ctor_get(x_257, 0); -lean_inc(x_258); -x_259 = lean_ctor_get(x_257, 1); -lean_inc(x_259); -lean_dec(x_257); -lean_inc(x_254); -x_260 = l_Std_Tactic_BVDecide_BVExpr_bitblast_go(x_254, x_258, x_256); -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); -x_263 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_263, 0, x_254); -lean_ctor_set(x_263, 1, x_259); -lean_ctor_set(x_263, 2, x_262); -x_264 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__40(x_1, x_261, x_263); +x_269 = l_Std_Tactic_BVDecide_BVExpr_bitblast_go(x_1, x_2, x_267); +x_270 = lean_ctor_get(x_269, 0); +lean_inc(x_270); +x_271 = lean_ctor_get(x_269, 1); +lean_inc(x_271); +lean_dec(x_269); +lean_inc(x_266); +x_272 = l_Std_Tactic_BVDecide_BVExpr_bitblast_go(x_266, x_270, x_268); +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); +x_275 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_275, 0, x_266); +lean_ctor_set(x_275, 1, x_271); +lean_ctor_set(x_275, 2, x_274); +x_276 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__42(x_1, x_273, x_275); lean_dec(x_1); -return x_264; +return x_276; } } } @@ -3415,32 +3814,42 @@ lean_dec(x_3); return x_12; } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRightConst_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___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_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv_signBranch___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__25___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv_signBranch___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__25(x_1, x_2, x_3); +lean_dec(x_3); +lean_dec(x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRightConst_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___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) { _start: { lean_object* x_8; -x_8 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRightConst_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__25(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRightConst_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__27(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); return x_8; } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRightConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__24___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRightConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__26___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRightConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__24(x_1, x_2, x_3); +x_4 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRightConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__26(x_1, x_2, x_3); lean_dec(x_3); lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateLeft_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___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_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateLeft_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___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) { _start: { lean_object* x_8; -x_8 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateLeft_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__27(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateLeft_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__29(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); @@ -3448,20 +3857,20 @@ lean_dec(x_1); return x_8; } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateLeft___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__26___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateLeft___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__28___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateLeft___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__26(x_1, x_2, x_3); +x_4 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateLeft___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__28(x_1, x_2, x_3); lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateRight_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___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_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateRight_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___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) { _start: { lean_object* x_8; -x_8 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateRight_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__29(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateRight_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__31(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); @@ -3469,20 +3878,20 @@ lean_dec(x_1); return x_8; } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateRight___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__28___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateRight___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__30___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateRight___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__28(x_1, x_2, x_3); +x_4 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastRotateRight___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__30(x_1, x_2, x_3); lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastArithShiftRightConst_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___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_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastArithShiftRightConst_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__33___boxed(lean_object* x_1, 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_Tactic_BVDecide_BVExpr_bitblast_blastArithShiftRightConst_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__31(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastArithShiftRightConst_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__33(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); @@ -3490,29 +3899,29 @@ lean_dec(x_1); return x_8; } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastArithShiftRightConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__30___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastArithShiftRightConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__32___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastArithShiftRightConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__30(x_1, x_2, x_3); +x_4 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastArithShiftRightConst___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__32(x_1, x_2, x_3); lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastAppend___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__32___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastAppend___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__34___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastAppend___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__32(x_1, x_2, x_3); +x_4 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastAppend___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__34(x_1, x_2, x_3); lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastReplicate_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___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_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastReplicate_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___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: { lean_object* x_8; -x_8 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastReplicate_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__34(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastReplicate_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__36(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); @@ -3520,21 +3929,21 @@ lean_dec(x_1); return x_8; } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastReplicate___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__33___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastReplicate___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__35___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastReplicate___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__33(x_1, x_2, x_3); +x_4 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastReplicate___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__35(x_1, x_2, x_3); lean_dec(x_3); lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSignExtend_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___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_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSignExtend_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___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, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; -x_9 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSignExtend_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__36(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSignExtend_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__38(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); @@ -3542,67 +3951,67 @@ lean_dec(x_1); return x_9; } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSignExtend___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__35___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSignExtend___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__37___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSignExtend___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__35(x_1, x_2, x_3); +x_4 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSignExtend___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__37(x_1, x_2, x_3); lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft_twoPowShift___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__38___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft_twoPowShift___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__40___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft_twoPowShift___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__38(x_1, x_2, x_3); +x_4 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft_twoPowShift___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__40(x_1, x_2, x_3); lean_dec(x_3); lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___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_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___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) { _start: { lean_object* x_7; -x_7 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__39(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__41(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__37___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__39___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__37(x_1, x_2, x_3); +x_4 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftLeft___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__39(x_1, x_2, x_3); lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight_twoPowShift___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__41___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight_twoPowShift___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__43___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight_twoPowShift___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__41(x_1, x_2, x_3); +x_4 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight_twoPowShift___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__43(x_1, x_2, x_3); lean_dec(x_3); lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__42___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__44___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; -x_7 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__42(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__44(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__40___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__42___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__40(x_1, x_2, x_3); +x_4 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastShiftRight___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__42(x_1, x_2, x_3); lean_dec(x_1); return x_4; } @@ -3615,6 +4024,7 @@ x_4 = l_Std_Tactic_BVDecide_BVExpr_bitblast_go(x_1, x_2, x_3); return x_4; } } +lean_object* initialize_Init_Data_AC(uint8_t builtin, lean_object*); lean_object* initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Impl_Var(uint8_t builtin, lean_object*); lean_object* initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Impl_Const(uint8_t builtin, lean_object*); lean_object* initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Impl_Operations_Not(uint8_t builtin, lean_object*); @@ -3631,11 +4041,15 @@ lean_object* initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Impl_Operati lean_object* initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Impl_Operations_Mul(uint8_t builtin, lean_object*); lean_object* initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Impl_Operations_Udiv(uint8_t builtin, lean_object*); lean_object* initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Impl_Operations_Umod(uint8_t builtin, lean_object*); +lean_object* initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Impl_Operations_Sdiv(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Impl_Expr(uint8_t builtin, lean_object* w) { lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; +res = initialize_Init_Data_AC(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); res = initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Impl_Var(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); @@ -3684,6 +4098,9 @@ lean_dec_ref(res); res = initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Impl_Operations_Umod(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +res = initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Impl_Operations_Sdiv(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Std_Tactic_BVDecide_BVExpr_bitblast_blastZeroExtend_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__2___closed__1 = _init_l_Std_Tactic_BVDecide_BVExpr_bitblast_blastZeroExtend_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__2___closed__1(); lean_mark_persistent(l_Std_Tactic_BVDecide_BVExpr_bitblast_blastZeroExtend_go___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__2___closed__1); l_Std_Tactic_BVDecide_BVPred_mkEq___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__8___closed__1 = _init_l_Std_Tactic_BVDecide_BVPred_mkEq___at_Std_Tactic_BVDecide_BVExpr_bitblast_go___spec__8___closed__1(); diff --git a/stage0/stdlib/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Impl/Operations/Sdiv.c b/stage0/stdlib/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Impl/Operations/Sdiv.c new file mode 100644 index 000000000000..9c8a1865d9cf --- /dev/null +++ b/stage0/stdlib/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Impl/Operations/Sdiv.c @@ -0,0 +1,468 @@ +// Lean compiler output +// Module: Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Sdiv +// Imports: Std.Sat.AIG.If Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Neg Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Udiv +#include +#if defined(__clang__) +#pragma clang diagnostic ignored "-Wunused-parameter" +#pragma clang diagnostic ignored "-Wunused-label" +#elif defined(__GNUC__) && !defined(__CLANG__) +#pragma GCC diagnostic ignored "-Wunused-parameter" +#pragma GCC diagnostic ignored "-Wunused-label" +#pragma GCC diagnostic ignored "-Wunused-but-set-variable" +#endif +#ifdef __cplusplus +extern "C" { +#endif +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv_signBranch___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_array_fget(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv(lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv_signBranch___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Std_Sat_AIG_RefVec_empty(lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t lean_nat_dec_eq(lean_object*, lean_object*); +lean_object* lean_nat_sub(lean_object*, lean_object*); +lean_object* l_Std_Sat_AIG_RefVec_ite___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastNeg___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv_signBranch(lean_object*); +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv_signBranch___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; 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_6 = lean_ctor_get(x_5, 0); +x_7 = lean_ctor_get(x_5, 1); +x_8 = lean_ctor_get(x_5, 2); +x_9 = lean_ctor_get(x_5, 3); +x_10 = lean_ctor_get(x_5, 4); +x_11 = lean_ctor_get(x_5, 5); +x_12 = lean_ctor_get(x_5, 6); +x_13 = lean_unsigned_to_nat(1u); +x_14 = lean_nat_sub(x_6, x_13); +x_15 = lean_array_fget(x_8, x_14); +x_16 = lean_array_fget(x_7, x_14); +lean_dec(x_14); +lean_inc(x_9); +lean_inc(x_10); +lean_inc(x_15); +x_17 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_17, 0, x_15); +lean_ctor_set(x_17, 1, x_10); +lean_ctor_set(x_17, 2, x_9); +lean_inc(x_2); +lean_inc(x_1); +x_18 = l_Std_Sat_AIG_RefVec_ite___rarg(x_1, x_2, x_3, 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); +lean_inc(x_11); +lean_inc(x_12); +x_21 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_21, 0, x_15); +lean_ctor_set(x_21, 1, x_12); +lean_ctor_set(x_21, 2, x_11); +lean_inc(x_2); +lean_inc(x_1); +x_22 = l_Std_Sat_AIG_RefVec_ite___rarg(x_1, x_2, x_3, x_19, 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_alloc_ctor(0, 3, 0); +lean_ctor_set(x_25, 0, x_16); +lean_ctor_set(x_25, 1, x_24); +lean_ctor_set(x_25, 2, x_20); +x_26 = l_Std_Sat_AIG_RefVec_ite___rarg(x_1, x_2, x_3, x_23, x_25); +return x_26; +} +} +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv_signBranch(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv_signBranch___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv_signBranch___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_Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv_signBranch___rarg(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_5); +lean_dec(x_3); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; uint8_t x_7; +x_6 = lean_unsigned_to_nat(0u); +x_7 = lean_nat_dec_eq(x_3, x_6); +if (x_7 == 0) +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_5); +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; uint8_t x_15; +x_9 = lean_ctor_get(x_5, 0); +x_10 = lean_ctor_get(x_5, 1); +lean_inc(x_9); +lean_inc(x_2); +lean_inc(x_1); +x_11 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastNeg___rarg(x_1, x_2, x_3, x_4, x_9); +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +lean_inc(x_10); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastNeg___rarg(x_1, x_2, x_3, x_12, x_10); +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 0) +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; 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; +x_16 = lean_ctor_get(x_14, 0); +x_17 = lean_ctor_get(x_14, 1); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_18 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv___rarg(x_1, x_2, x_3, x_16, x_5); +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +x_20 = lean_ctor_get(x_18, 1); +lean_inc(x_20); +lean_dec(x_18); +lean_inc(x_17); +lean_inc(x_9); +lean_ctor_set(x_14, 0, x_9); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_21 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv___rarg(x_1, x_2, x_3, x_19, x_14); +x_22 = lean_ctor_get(x_21, 0); +lean_inc(x_22); +x_23 = lean_ctor_get(x_21, 1); +lean_inc(x_23); +lean_dec(x_21); +lean_inc(x_2); +lean_inc(x_1); +x_24 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastNeg___rarg(x_1, x_2, x_3, x_22, x_23); +x_25 = lean_ctor_get(x_24, 0); +lean_inc(x_25); +x_26 = lean_ctor_get(x_24, 1); +lean_inc(x_26); +lean_dec(x_24); +lean_inc(x_10); +lean_inc(x_13); +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_13); +lean_ctor_set(x_27, 1, x_10); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_28 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv___rarg(x_1, x_2, x_3, x_25, 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_2); +lean_inc(x_1); +x_31 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastNeg___rarg(x_1, x_2, x_3, x_29, x_30); +x_32 = lean_ctor_get(x_31, 0); +lean_inc(x_32); +x_33 = lean_ctor_get(x_31, 1); +lean_inc(x_33); +lean_dec(x_31); +x_34 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_34, 0, x_13); +lean_ctor_set(x_34, 1, x_17); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_35 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv___rarg(x_1, x_2, x_3, x_32, 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); +lean_inc(x_3); +x_38 = lean_alloc_ctor(0, 7, 0); +lean_ctor_set(x_38, 0, x_3); +lean_ctor_set(x_38, 1, x_9); +lean_ctor_set(x_38, 2, x_10); +lean_ctor_set(x_38, 3, x_20); +lean_ctor_set(x_38, 4, x_26); +lean_ctor_set(x_38, 5, x_33); +lean_ctor_set(x_38, 6, x_37); +x_39 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv_signBranch___rarg(x_1, x_2, x_3, x_36, x_38); +lean_dec(x_38); +lean_dec(x_3); +return x_39; +} +else +{ +lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; +x_40 = lean_ctor_get(x_14, 0); +x_41 = lean_ctor_get(x_14, 1); +lean_inc(x_41); +lean_inc(x_40); +lean_dec(x_14); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_42 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv___rarg(x_1, x_2, x_3, x_40, x_5); +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_41); +lean_inc(x_9); +x_45 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_45, 0, x_9); +lean_ctor_set(x_45, 1, x_41); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_46 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv___rarg(x_1, x_2, x_3, x_43, 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); +lean_inc(x_2); +lean_inc(x_1); +x_49 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastNeg___rarg(x_1, x_2, x_3, x_47, x_48); +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_10); +lean_inc(x_13); +x_52 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_52, 0, x_13); +lean_ctor_set(x_52, 1, x_10); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_53 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv___rarg(x_1, x_2, x_3, x_50, 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_2); +lean_inc(x_1); +x_56 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastNeg___rarg(x_1, x_2, x_3, x_54, x_55); +x_57 = lean_ctor_get(x_56, 0); +lean_inc(x_57); +x_58 = lean_ctor_get(x_56, 1); +lean_inc(x_58); +lean_dec(x_56); +x_59 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_59, 0, x_13); +lean_ctor_set(x_59, 1, x_41); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_60 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv___rarg(x_1, x_2, x_3, x_57, 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); +lean_inc(x_3); +x_63 = lean_alloc_ctor(0, 7, 0); +lean_ctor_set(x_63, 0, x_3); +lean_ctor_set(x_63, 1, x_9); +lean_ctor_set(x_63, 2, x_10); +lean_ctor_set(x_63, 3, x_44); +lean_ctor_set(x_63, 4, x_51); +lean_ctor_set(x_63, 5, x_58); +lean_ctor_set(x_63, 6, x_62); +x_64 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv_signBranch___rarg(x_1, x_2, x_3, x_61, x_63); +lean_dec(x_63); +lean_dec(x_3); +return x_64; +} +} +else +{ +lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; +x_65 = lean_ctor_get(x_5, 0); +x_66 = lean_ctor_get(x_5, 1); +lean_inc(x_66); +lean_inc(x_65); +lean_dec(x_5); +lean_inc(x_65); +lean_inc(x_2); +lean_inc(x_1); +x_67 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastNeg___rarg(x_1, x_2, x_3, x_4, x_65); +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_66); +lean_inc(x_2); +lean_inc(x_1); +x_70 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastNeg___rarg(x_1, x_2, x_3, x_68, x_66); +x_71 = lean_ctor_get(x_70, 0); +lean_inc(x_71); +x_72 = lean_ctor_get(x_70, 1); +lean_inc(x_72); +if (lean_is_exclusive(x_70)) { + lean_ctor_release(x_70, 0); + lean_ctor_release(x_70, 1); + x_73 = x_70; +} else { + lean_dec_ref(x_70); + x_73 = lean_box(0); +} +lean_inc(x_66); +lean_inc(x_65); +x_74 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_74, 0, x_65); +lean_ctor_set(x_74, 1, x_66); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_75 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv___rarg(x_1, x_2, x_3, x_71, x_74); +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_72); +lean_inc(x_65); +if (lean_is_scalar(x_73)) { + x_78 = lean_alloc_ctor(0, 2, 0); +} else { + x_78 = x_73; +} +lean_ctor_set(x_78, 0, x_65); +lean_ctor_set(x_78, 1, x_72); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_79 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv___rarg(x_1, x_2, x_3, x_76, 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); +lean_inc(x_2); +lean_inc(x_1); +x_82 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastNeg___rarg(x_1, x_2, x_3, x_80, 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); +lean_inc(x_66); +lean_inc(x_69); +x_85 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_85, 0, x_69); +lean_ctor_set(x_85, 1, x_66); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_86 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv___rarg(x_1, x_2, x_3, x_83, x_85); +x_87 = lean_ctor_get(x_86, 0); +lean_inc(x_87); +x_88 = lean_ctor_get(x_86, 1); +lean_inc(x_88); +lean_dec(x_86); +lean_inc(x_2); +lean_inc(x_1); +x_89 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastNeg___rarg(x_1, x_2, x_3, x_87, 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); +x_92 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_92, 0, x_69); +lean_ctor_set(x_92, 1, x_72); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_93 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastUdiv___rarg(x_1, x_2, x_3, x_90, 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); +lean_inc(x_3); +x_96 = lean_alloc_ctor(0, 7, 0); +lean_ctor_set(x_96, 0, x_3); +lean_ctor_set(x_96, 1, x_65); +lean_ctor_set(x_96, 2, x_66); +lean_ctor_set(x_96, 3, x_77); +lean_ctor_set(x_96, 4, x_84); +lean_ctor_set(x_96, 5, x_91); +lean_ctor_set(x_96, 6, x_95); +x_97 = l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv_signBranch___rarg(x_1, x_2, x_3, x_94, x_96); +lean_dec(x_96); +lean_dec(x_3); +return x_97; +} +} +else +{ +lean_object* x_98; lean_object* x_99; +lean_dec(x_5); +lean_dec(x_3); +x_98 = l_Std_Sat_AIG_RefVec_empty(lean_box(0), x_1, x_2, x_4); +lean_dec(x_2); +lean_dec(x_1); +x_99 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_99, 0, x_4); +lean_ctor_set(x_99, 1, x_98); +return x_99; +} +} +} +LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv___rarg), 5, 0); +return x_2; +} +} +lean_object* initialize_Std_Sat_AIG_If(uint8_t builtin, lean_object*); +lean_object* initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Impl_Operations_Neg(uint8_t builtin, lean_object*); +lean_object* initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Impl_Operations_Udiv(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Impl_Operations_Sdiv(uint8_t builtin, lean_object* w) { +lean_object * res; +if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); +_G_initialized = true; +res = initialize_Std_Sat_AIG_If(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Impl_Operations_Neg(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Impl_Operations_Udiv(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +return lean_io_result_mk_ok(lean_box(0)); +} +#ifdef __cplusplus +} +#endif diff --git a/stage0/stdlib/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Lemmas/Expr.c b/stage0/stdlib/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Lemmas/Expr.c index 86ffb5aa0119..99d8df7cf6cb 100644 --- a/stage0/stdlib/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Lemmas/Expr.c +++ b/stage0/stdlib/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Lemmas/Expr.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Expr -// Imports: Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Basic Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Const Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Var Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.Not Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.ShiftLeft Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.ShiftRight Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.Add Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.ZeroExtend Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.Append Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.Replicate Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.Extract Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.RotateLeft Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.RotateRight Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.SignExtend Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.Mul Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.Udiv Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.Umod Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Expr +// Imports: Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Basic Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Const Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Var Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.Not Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.ShiftLeft Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.ShiftRight Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.Add Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.ZeroExtend Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.Append Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.Replicate Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.Extract Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.RotateLeft Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.RotateRight Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.SignExtend Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.Mul Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.Udiv Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.Umod Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.Sdiv Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Expr #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -290,6 +290,7 @@ lean_object* initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Lemmas_Opera lean_object* initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Lemmas_Operations_Mul(uint8_t builtin, lean_object*); lean_object* initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Lemmas_Operations_Udiv(uint8_t builtin, lean_object*); lean_object* initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Lemmas_Operations_Umod(uint8_t builtin, lean_object*); +lean_object* initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Lemmas_Operations_Sdiv(uint8_t builtin, lean_object*); lean_object* initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Impl_Expr(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Lemmas_Expr(uint8_t builtin, lean_object* w) { @@ -347,6 +348,9 @@ lean_dec_ref(res); res = initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Lemmas_Operations_Umod(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +res = initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Lemmas_Operations_Sdiv(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); res = initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Impl_Expr(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Lemmas/Operations/Sdiv.c b/stage0/stdlib/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Lemmas/Operations/Sdiv.c new file mode 100644 index 000000000000..16d6575276e6 --- /dev/null +++ b/stage0/stdlib/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Lemmas/Operations/Sdiv.c @@ -0,0 +1,99 @@ +// Lean compiler output +// Module: Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.Sdiv +// Imports: Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.Udiv Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Operations.Neg Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Sdiv Std.Tactic.BVDecide.Normalize.BitVec +#include +#if defined(__clang__) +#pragma clang diagnostic ignored "-Wunused-parameter" +#pragma clang diagnostic ignored "-Wunused-label" +#elif defined(__GNUC__) && !defined(__CLANG__) +#pragma GCC diagnostic ignored "-Wunused-parameter" +#pragma GCC diagnostic ignored "-Wunused-label" +#pragma GCC diagnostic ignored "-Wunused-but-set-variable" +#endif +#ifdef __cplusplus +extern "C" { +#endif +LEAN_EXPORT lean_object* l___private_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Lemmas_Operations_Sdiv_0__Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv_denote__signBranch_match__1_splitter___rarg(uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Lemmas_Operations_Sdiv_0__Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv_denote__signBranch_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Lemmas_Operations_Sdiv_0__Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv_denote__signBranch_match__1_splitter(lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Lemmas_Operations_Sdiv_0__Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv_denote__signBranch_match__1_splitter___rarg(uint8_t x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +if (x_1 == 0) +{ +if (x_2 == 0) +{ +lean_inc(x_3); +return x_3; +} +else +{ +lean_inc(x_4); +return x_4; +} +} +else +{ +if (x_2 == 0) +{ +lean_inc(x_5); +return x_5; +} +else +{ +lean_inc(x_6); +return x_6; +} +} +} +} +LEAN_EXPORT lean_object* l___private_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Lemmas_Operations_Sdiv_0__Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv_denote__signBranch_match__1_splitter(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l___private_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Lemmas_Operations_Sdiv_0__Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv_denote__signBranch_match__1_splitter___rarg___boxed), 6, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Lemmas_Operations_Sdiv_0__Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv_denote__signBranch_match__1_splitter___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +uint8_t x_7; uint8_t x_8; lean_object* x_9; +x_7 = lean_unbox(x_1); +lean_dec(x_1); +x_8 = lean_unbox(x_2); +lean_dec(x_2); +x_9 = l___private_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Lemmas_Operations_Sdiv_0__Std_Tactic_BVDecide_BVExpr_bitblast_blastSdiv_denote__signBranch_match__1_splitter___rarg(x_7, x_8, x_3, x_4, x_5, x_6); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_9; +} +} +lean_object* initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Lemmas_Operations_Udiv(uint8_t builtin, lean_object*); +lean_object* initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Lemmas_Operations_Neg(uint8_t builtin, lean_object*); +lean_object* initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Impl_Operations_Sdiv(uint8_t builtin, lean_object*); +lean_object* initialize_Std_Tactic_BVDecide_Normalize_BitVec(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Lemmas_Operations_Sdiv(uint8_t builtin, lean_object* w) { +lean_object * res; +if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); +_G_initialized = true; +res = initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Lemmas_Operations_Udiv(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Lemmas_Operations_Neg(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Impl_Operations_Sdiv(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Std_Tactic_BVDecide_Normalize_BitVec(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +return lean_io_result_mk_ok(lean_box(0)); +} +#ifdef __cplusplus +} +#endif diff --git a/stage0/stdlib/Std/Tactic/BVDecide/LRAT/Internal/Clause.c b/stage0/stdlib/Std/Tactic/BVDecide/LRAT/Internal/Clause.c index 4535d5388005..207eba069d5a 100644 --- a/stage0/stdlib/Std/Tactic/BVDecide/LRAT/Internal/Clause.c +++ b/stage0/stdlib/Std/Tactic/BVDecide/LRAT/Internal/Clause.c @@ -44,7 +44,6 @@ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Std_Tactic_BVDecide_LRAT LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Std_Tactic_BVDecide_LRAT_Internal_DefaultClause_ofArray___spec__2(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_LRAT_Internal_DefaultClause_reduce__fold__fn___boxed(lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_LRAT_Internal_DefaultClause_unit___rarg(lean_object*); -LEAN_EXPORT lean_object* l___private_Std_Tactic_BVDecide_LRAT_Internal_Clause_0__List_getLast_x3f_match__1_splitter(lean_object*, lean_object*); uint8_t l_List_any___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_eraseTR_go___at_Std_Tactic_BVDecide_LRAT_Internal_DefaultClause_delete___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_LRAT_Internal_DefaultClause_isUnit___rarg(lean_object*); @@ -63,7 +62,6 @@ LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_LRAT_Internal_DefaultClause_empty LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_LRAT_Internal_DefaultClause_toList(lean_object*); LEAN_EXPORT lean_object* l_List_toString___at_Std_Tactic_BVDecide_LRAT_Internal_instToStringDefaultClause___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_LRAT_Internal_DefaultClause_insert___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Std_Tactic_BVDecide_LRAT_Internal_Clause_0__List_getLast_x3f_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_LRAT_Internal_DefaultClause_reduce___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_LRAT_Internal_Clause_instDecidableEvalLiteral___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at_Std_Tactic_BVDecide_LRAT_Internal_instToStringDefaultClause___spec__3___boxed(lean_object*, lean_object*, lean_object*); @@ -72,7 +70,6 @@ LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_LRAT_Internal_DefaultClause_unit_ LEAN_EXPORT uint8_t l_List_elem___at_Std_Tactic_BVDecide_LRAT_Internal_DefaultClause_insert___spec__2(lean_object*, lean_object*, lean_object*); lean_object* l_outOfBounds___rarg(lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_LRAT_Internal_DefaultClause_instClausePosFin(lean_object*); -LEAN_EXPORT lean_object* l___private_Std_Tactic_BVDecide_LRAT_Internal_Clause_0__List_getLast_x3f_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_LRAT_Internal_DefaultClause_empty(lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_LRAT_Internal_DefaultClause_toList___boxed(lean_object*); LEAN_EXPORT lean_object* l_List_toString___at_Std_Tactic_BVDecide_LRAT_Internal_instToStringDefaultClause___spec__1___boxed(lean_object*, lean_object*); @@ -816,45 +813,6 @@ lean_dec(x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Std_Tactic_BVDecide_LRAT_Internal_Clause_0__List_getLast_x3f_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -if (lean_obj_tag(x_1) == 0) -{ -lean_dec(x_3); -lean_inc(x_2); -return x_2; -} -else -{ -lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_4 = lean_ctor_get(x_1, 0); -lean_inc(x_4); -x_5 = lean_ctor_get(x_1, 1); -lean_inc(x_5); -lean_dec(x_1); -x_6 = lean_apply_2(x_3, x_4, x_5); -return x_6; -} -} -} -LEAN_EXPORT lean_object* l___private_Std_Tactic_BVDecide_LRAT_Internal_Clause_0__List_getLast_x3f_match__1_splitter(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l___private_Std_Tactic_BVDecide_LRAT_Internal_Clause_0__List_getLast_x3f_match__1_splitter___rarg___boxed), 3, 0); -return x_3; -} -} -LEAN_EXPORT lean_object* l___private_Std_Tactic_BVDecide_LRAT_Internal_Clause_0__List_getLast_x3f_match__1_splitter___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l___private_Std_Tactic_BVDecide_LRAT_Internal_Clause_0__List_getLast_x3f_match__1_splitter___rarg(x_1, x_2, x_3); -lean_dec(x_2); -return x_4; -} -} LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_LRAT_Internal_DefaultClause_empty(lean_object* x_1) { _start: { diff --git a/tests/bench/big_do.lean b/tests/bench/big_do.lean new file mode 100644 index 000000000000..41319f1aaa66 --- /dev/null +++ b/tests/bench/big_do.lean @@ -0,0 +1,459 @@ +/-! +This benchmark exercises +* general elaboration, likely from many nested lambdas +* code generation, ditto +-/ + +set_option maxRecDepth 10000 + +def addALot (x: Nat) : StateM Nat Nat := do + set x + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + modifyGet (λ y => ((), y + x)) + let y <- get + pure y + +#eval StateT.run' (addALot 2) 0 diff --git a/tests/bench/big_omega.lean b/tests/bench/big_omega.lean new file mode 100644 index 000000000000..138db4cda456 --- /dev/null +++ b/tests/bench/big_omega.lean @@ -0,0 +1,40 @@ +/-! +This benchmark exercises `omega` in a way that creates a big proof, exercising `instantiateMVars` +and `shareCommonPreDefs` as well. In particular, running it with `internal.cmdlineSnapshots=false`, +like the language server does, uncovered a significant slowdown in `instantiateMVars` (#5614). +-/ + +set_option maxHeartbeats 0 +theorem memcpy_extracted_2 (six0 s0x0 : BitVec 64) +(h_six0_nonzero : six0 ≠ 0) +(h_s0x1 : s0x1 + 16#64 * (s0x0 - six0) + 16#64 = s0x1 + 16#64 * (s0x0 - (six0 - 1#64))) +(h_s0x2 : s0x2 + 16#64 * (s0x0 - six0) + 16#64 = s0x2 + 16#64 * (s0x0 - (six0 - 1#64))) +(h_assert_1 : six0 ≤ s0x0) +(h_assert_3 : six1 = s0x1 + 16#64 * (s0x0 - six0)) +(h_assert_4 : six2 = s0x2 + 16#64 * (s0x0 - six0)) +(n : Nat) +(addr : BitVec 64) +(h_le : (s0x0 - (six0 - 1#64)).toNat ≤ s0x0.toNat) +(h_upper_bound : addr.toNat + n ≤ 2 ^ 64) +(h_upper_bound₂ : s0x2.toNat + s0x0.toNat * 16 ≤ 2 ^ 64) +(h_upper_bound₃ : s0x2.toNat + (16#64 * (s0x0 - (six0 - 1#64))).toNat ≤ 2 ^ 64) +(h_width_lt : (16#64).toNat * (s0x0 - (six0 - 1#64)).toNat < 2 ^ 64) +(hmemSeparate_omega : s0x1.toNat + s0x0.toNat * 16 ≤ 2 ^ 64 ∧ + s0x2.toNat + s0x0.toNat * 16 ≤ 2 ^ 64 ∧ + (s0x1.toNat + s0x0.toNat * 16 ≤ s0x2.toNat ∨ s0x1.toNat ≥ s0x2.toNat + s0x0.toNat * 16)) +(hmemLegal_omega : s0x1.toNat + s0x0.toNat * 16 ≤ 2 ^ 64) +(hmemLegal_omega : s0x2.toNat + s0x0.toNat * 16 ≤ 2 ^ 64) +(hmemSeparate_omega : s0x2.toNat + 16 % 2 ^ 64 * ((2 ^ 64 - (2 ^ 64 - 1 % 2 ^ 64 + six0.toNat) % 2 ^ 64 + s0x0.toNat) % 2 ^ 64) % 2 ^ 64 ≤ + 2 ^ 64 ∧ + addr.toNat + n ≤ 2 ^ 64 ∧ + (s0x2.toNat + + 16 % 2 ^ 64 * ((2 ^ 64 - (2 ^ 64 - 1 % 2 ^ 64 + six0.toNat) % 2 ^ 64 + s0x0.toNat) % 2 ^ 64) % 2 ^ 64 ≤ + addr.toNat ∨ + s0x2.toNat ≥ addr.toNat + n)) +(hmemLegal_omega : s0x2.toNat + 16 % 2 ^ 64 * ((2 ^ 64 - (2 ^ 64 - 1 % 2 ^ 64 + six0.toNat) % 2 ^ 64 + s0x0.toNat) % 2 ^ 64) % 2 ^ 64 ≤ + 2 ^ 64) +(hmemLegal_omega : addr.toNat + n ≤ 2 ^ 64) : + s0x2.toNat + (16#64 * (s0x0 - six0)).toNat ≤ 2 ^ 64 ∧ + addr.toNat + n ≤ 2 ^ 64 ∧ + (s0x2.toNat + (16#64 * (s0x0 - six0)).toNat ≤ addr.toNat ∨ s0x2.toNat ≥ addr.toNat + n) := by + bv_omega diff --git a/tests/bench/speedcenter.exec.velcom.yaml b/tests/bench/speedcenter.exec.velcom.yaml index ce08a96f6a0d..b970bde71eae 100644 --- a/tests/bench/speedcenter.exec.velcom.yaml +++ b/tests/bench/speedcenter.exec.velcom.yaml @@ -362,3 +362,21 @@ run_config: <<: *time cmd: lean bv_decide_inequality.lean +- attributes: + description: big_do + tags: [fast] + run_config: + <<: *time + cmd: lean big_do.lean +- attributes: + description: big_omega.lean + tags: [fast] + run_config: + <<: *time + cmd: lean big_omega.lean +- attributes: + description: big_omega.lean MT + tags: [fast] + run_config: + <<: *time + cmd: lean big_omega.lean -Dinternal.cmdlineSnapshots=false diff --git a/tests/lean/1021.lean.expected.out b/tests/lean/1021.lean.expected.out index aef0080bffb6..d7aee5388923 100644 --- a/tests/lean/1021.lean.expected.out +++ b/tests/lean/1021.lean.expected.out @@ -1,7 +1,7 @@ some { range := - { pos := { line := 202, column := 42 }, charUtf16 := 42, endPos := { line := 208, column := 31 }, + { pos := { line := 202, column := 0 }, charUtf16 := 0, endPos := { line := 208, column := 31 }, endCharUtf16 := 31 }, selectionRange := { pos := { line := 202, column := 46 }, charUtf16 := 46, endPos := { line := 202, column := 58 }, diff --git a/tests/lean/4845.lean b/tests/lean/4845.lean new file mode 100644 index 000000000000..f22af6301e5e --- /dev/null +++ b/tests/lean/4845.lean @@ -0,0 +1,12 @@ +/-! + Generalize should not try to abstract the variable from hypotheses that are + implementation details. -/ + +/-! + In this case, generalize tries to revert the lemma being defined to generalize + the 0 in it. -/ + +example : 0 = 0 → True := by + intro H; generalize _H : 0 = z at * + trace_state + constructor diff --git a/tests/lean/4845.lean.expected.out b/tests/lean/4845.lean.expected.out new file mode 100644 index 000000000000..7a20a98e3073 --- /dev/null +++ b/tests/lean/4845.lean.expected.out @@ -0,0 +1,4 @@ +z : Nat +_H : 0 = z +H : z = z +⊢ True diff --git a/tests/lean/classBadOutParam.lean.expected.out b/tests/lean/classBadOutParam.lean.expected.out index 705f3cc8921e..036aff2631fb 100644 --- a/tests/lean/classBadOutParam.lean.expected.out +++ b/tests/lean/classBadOutParam.lean.expected.out @@ -1 +1 @@ -classBadOutParam.lean:3:1-3:4: error: invalid class, parameter #2 depends on `outParam`, but it is not an `outParam` +classBadOutParam.lean:2:6-2:8: error: invalid class, parameter #2 depends on `outParam`, but it is not an `outParam` diff --git a/tests/lean/delabOverApp.lean.expected.out b/tests/lean/delabOverApp.lean.expected.out index 43157f618050..db68ae147eee 100644 --- a/tests/lean/delabOverApp.lean.expected.out +++ b/tests/lean/delabOverApp.lean.expected.out @@ -3,4 +3,4 @@ f +' g : Nat → Nat f * g : Nat → Nat (f * g) 1 : Nat mul f g : Nat → Nat -mul f g 1 : Nat +mul f g (@OfNat.ofNat Nat 1 (instOfNatNat 1)) : Nat diff --git a/tests/lean/interactive/completion2.lean.expected.out b/tests/lean/interactive/completion2.lean.expected.out index 6e34e1033472..3f9aafd094c0 100644 --- a/tests/lean/interactive/completion2.lean.expected.out +++ b/tests/lean/interactive/completion2.lean.expected.out @@ -3,7 +3,7 @@ {"items": [{"sortText": "0", "label": "ax1", - "kind": 3, + "kind": 23, "data": {"params": {"textDocument": {"uri": "file:///completion2.lean"}, @@ -11,7 +11,7 @@ "id": {"const": {"declName": "Foo.Bla.ax1"}}}}, {"sortText": "1", "label": "ex1", - "kind": 3, + "kind": 23, "data": {"params": {"textDocument": {"uri": "file:///completion2.lean"}, @@ -19,7 +19,7 @@ "id": {"const": {"declName": "Foo.Bla.ex1"}}}}, {"sortText": "2", "label": "ex2", - "kind": 3, + "kind": 23, "data": {"params": {"textDocument": {"uri": "file:///completion2.lean"}, @@ -27,7 +27,7 @@ "id": {"const": {"declName": "Foo.Bla.ex2"}}}}, {"sortText": "3", "label": "ex3", - "kind": 3, + "kind": 23, "data": {"params": {"textDocument": {"uri": "file:///completion2.lean"}, @@ -39,7 +39,7 @@ {"items": [{"sortText": "0", "label": "ax1", - "kind": 3, + "kind": 23, "data": {"params": {"textDocument": {"uri": "file:///completion2.lean"}, @@ -47,7 +47,7 @@ "id": {"const": {"declName": "Foo.Bla.ax1"}}}}, {"sortText": "1", "label": "ex1", - "kind": 3, + "kind": 23, "data": {"params": {"textDocument": {"uri": "file:///completion2.lean"}, @@ -55,7 +55,7 @@ "id": {"const": {"declName": "Foo.Bla.ex1"}}}}, {"sortText": "2", "label": "ex2", - "kind": 3, + "kind": 23, "data": {"params": {"textDocument": {"uri": "file:///completion2.lean"}, @@ -63,7 +63,7 @@ "id": {"const": {"declName": "Foo.Bla.ex2"}}}}, {"sortText": "3", "label": "ex3", - "kind": 3, + "kind": 23, "data": {"params": {"textDocument": {"uri": "file:///completion2.lean"}, @@ -75,7 +75,7 @@ {"items": [{"sortText": "0", "label": "ax1", - "kind": 3, + "kind": 23, "data": {"params": {"textDocument": {"uri": "file:///completion2.lean"}, @@ -83,7 +83,7 @@ "id": {"const": {"declName": "Foo.Bla.ax1"}}}}, {"sortText": "1", "label": "ex1", - "kind": 3, + "kind": 23, "data": {"params": {"textDocument": {"uri": "file:///completion2.lean"}, @@ -91,7 +91,7 @@ "id": {"const": {"declName": "Foo.Bla.ex1"}}}}, {"sortText": "2", "label": "ex2", - "kind": 3, + "kind": 23, "data": {"params": {"textDocument": {"uri": "file:///completion2.lean"}, @@ -99,7 +99,7 @@ "id": {"const": {"declName": "Foo.Bla.ex2"}}}}, {"sortText": "3", "label": "ex3", - "kind": 3, + "kind": 23, "data": {"params": {"textDocument": {"uri": "file:///completion2.lean"}, @@ -111,7 +111,7 @@ {"items": [{"sortText": "0", "label": "ex1", - "kind": 3, + "kind": 23, "data": {"params": {"textDocument": {"uri": "file:///completion2.lean"}, @@ -119,7 +119,7 @@ "id": {"const": {"declName": "Foo.Bla.ex1"}}}}, {"sortText": "1", "label": "ex2", - "kind": 3, + "kind": 23, "data": {"params": {"textDocument": {"uri": "file:///completion2.lean"}, @@ -127,7 +127,7 @@ "id": {"const": {"declName": "Foo.Bla.ex2"}}}}, {"sortText": "2", "label": "ex3", - "kind": 3, + "kind": 23, "data": {"params": {"textDocument": {"uri": "file:///completion2.lean"}, diff --git a/tests/lean/interactive/completionFallback.lean.expected.out b/tests/lean/interactive/completionFallback.lean.expected.out index 7cd2e288a01b..0d524243dc7b 100644 --- a/tests/lean/interactive/completionFallback.lean.expected.out +++ b/tests/lean/interactive/completionFallback.lean.expected.out @@ -55,7 +55,7 @@ {"items": [{"sortText": "0", "label": "ha", - "kind": 5, + "kind": 23, "data": {"params": {"textDocument": {"uri": "file:///completionFallback.lean"}, @@ -63,7 +63,7 @@ "id": {"const": {"declName": "CustomAnd.ha"}}}}, {"sortText": "1", "label": "hb", - "kind": 5, + "kind": 23, "data": {"params": {"textDocument": {"uri": "file:///completionFallback.lean"}, diff --git a/tests/lean/interactive/completionPrv.lean.expected.out b/tests/lean/interactive/completionPrv.lean.expected.out index 6c62ec4e392b..ac03b62acc90 100644 --- a/tests/lean/interactive/completionPrv.lean.expected.out +++ b/tests/lean/interactive/completionPrv.lean.expected.out @@ -31,7 +31,7 @@ "id": {"const": {"declName": "instToBoolBool"}}}}, {"sortText": "2", "label": "BitVec.getElem_ofBoolListBE", - "kind": 3, + "kind": 23, "data": {"params": {"textDocument": {"uri": "file:///completionPrv.lean"}, @@ -39,7 +39,7 @@ "id": {"const": {"declName": "BitVec.getElem_ofBoolListBE"}}}}, {"sortText": "3", "label": "BitVec.getLsbD_ofBoolListBE", - "kind": 3, + "kind": 23, "data": {"params": {"textDocument": {"uri": "file:///completionPrv.lean"}, @@ -47,7 +47,7 @@ "id": {"const": {"declName": "BitVec.getLsbD_ofBoolListBE"}}}}, {"sortText": "4", "label": "BitVec.getMsbD_ofBoolListBE", - "kind": 3, + "kind": 23, "data": {"params": {"textDocument": {"uri": "file:///completionPrv.lean"}, @@ -55,7 +55,7 @@ "id": {"const": {"declName": "BitVec.getMsbD_ofBoolListBE"}}}}, {"sortText": "5", "label": "BitVec.ofBool_and_ofBool", - "kind": 3, + "kind": 23, "data": {"params": {"textDocument": {"uri": "file:///completionPrv.lean"}, @@ -63,7 +63,7 @@ "id": {"const": {"declName": "BitVec.ofBool_and_ofBool"}}}}, {"sortText": "6", "label": "BitVec.ofBool_or_ofBool", - "kind": 3, + "kind": 23, "data": {"params": {"textDocument": {"uri": "file:///completionPrv.lean"}, @@ -71,7 +71,7 @@ "id": {"const": {"declName": "BitVec.ofBool_or_ofBool"}}}}, {"sortText": "7", "label": "BitVec.ofBool_xor_ofBool", - "kind": 3, + "kind": 23, "data": {"params": {"textDocument": {"uri": "file:///completionPrv.lean"}, diff --git a/tests/lean/interactive/travellingCompletions.lean.expected.out b/tests/lean/interactive/travellingCompletions.lean.expected.out index 46409f6f6b53..15c1f442e7d0 100644 --- a/tests/lean/interactive/travellingCompletions.lean.expected.out +++ b/tests/lean/interactive/travellingCompletions.lean.expected.out @@ -39,7 +39,7 @@ {"items": [{"sortText": "0", "label": "continuousAdd", - "kind": 3, + "kind": 23, "data": {"params": {"textDocument": {"uri": "file:///travellingCompletions.lean"}, @@ -47,7 +47,7 @@ "id": {"const": {"declName": "Prod.continuousAdd"}}}}, {"sortText": "1", "label": "continuousSMul", - "kind": 3, + "kind": 23, "data": {"params": {"textDocument": {"uri": "file:///travellingCompletions.lean"}, diff --git a/tests/lean/mvarAtDefaultValue.lean.expected.out b/tests/lean/mvarAtDefaultValue.lean.expected.out index 1d624efc9b4a..fe108527cb37 100644 --- a/tests/lean/mvarAtDefaultValue.lean.expected.out +++ b/tests/lean/mvarAtDefaultValue.lean.expected.out @@ -1,4 +1,14 @@ -mvarAtDefaultValue.lean:5:2-5:3: error: invalid default value for field, it contains metavariables +mvarAtDefaultValue.lean:5:7-5:8: error: don't know how to synthesize placeholder +context: +toA : A +x : Nat := toA.x +⊢ Nat +mvarAtDefaultValue.lean:5:2-5:3: error: invalid default value for field 'x', it contains metavariables ?m -mvarAtDefaultValue.lean:8:2-8:3: error: invalid default value for field, it contains metavariables +mvarAtDefaultValue.lean:8:7-8:8: error: don't know how to synthesize placeholder +context: +toA : A +x : Nat := toA.x +⊢ Nat +mvarAtDefaultValue.lean:8:2-8:3: error: invalid default value for field 'x', it contains metavariables ?m + 1 diff --git a/tests/lean/run/2186.lean b/tests/lean/run/2186.lean new file mode 100644 index 000000000000..3718e76f4f4d --- /dev/null +++ b/tests/lean/run/2186.lean @@ -0,0 +1,78 @@ +/-! +# Regression tests for #2186 + +https://github.com/leanprover/lean4/issues/2186 +-/ + +/-! +Minimization of the issue. The default value to `bar` wasn't working +because the default value of `bar` was `fun (_ : p) => trivial`, +and `p` (which in the default value itself appears as a projection) wasn't being reduced. +-/ +namespace Test1 + +structure A (α : Type u) where + p : Prop + bar : p → True + +structure B (α : Type _) extends A α where + bar _ := trivial + +-- Previously this needed `bar` to be specified +example : B α where + p := False + +end Test1 + +/-! +Tests from the issue. +-/ +namespace Test2 +variable (α : Type _) + +-- First example +structure A extends LE α where + foo : True +structure B extends LE α where + bar : ∀ a b : α, a ≤ b → True +structure C extends A α, B α + +structure D extends C α where + foo := trivial +structure E extends C α where + bar _ _ _ := trivial + +-- Always worked +example : D α where + le := Eq + bar _ _ _ := trivial +-- Didn't work +example : E α where + le := Eq + foo := trivial + +-- Second example +structure X where + transform : α → α + +structure A₁ extends X α where + foo : True +structure B₁ extends X α where + bar : ∀ a, transform a = transform (transform a) → True +structure C₁ extends A₁ α, B₁ α + +structure D₁ extends C₁ α where + foo := trivial +structure E₁ extends C₁ α where + bar _ _ := trivial + +-- Always worked +example : D₁ α where + transform := id + bar := fun _ _ => trivial +-- Didn't work +example : E₁ α where + transform := id + foo := trivial + +end Test2 diff --git a/tests/lean/run/3146.lean b/tests/lean/run/3146.lean new file mode 100644 index 000000000000..1facd54b126a --- /dev/null +++ b/tests/lean/run/3146.lean @@ -0,0 +1,13 @@ +/- + Verifies that `let`-bodies are reduced accordingly when trying to construct default fields. + Fixes `#3146` +-/ + +def Product (m₁ : Type → Type) (m₂ : Type → Type) (α : Type) := m₁ α × m₂ α + +instance [Monad m₁] [Monad m₂] : Monad (Product m₁ m₂) where + pure x := (pure x, pure x) + bind o f := + let y₁ := do f (← o.1) |>.1 + let y₂ := do f (← o.2) |>.2 + (y₁, y₂) diff --git a/tests/lean/run/3146.lean.expected.out b/tests/lean/run/3146.lean.expected.out new file mode 100644 index 000000000000..e69de29bb2d1 diff --git a/tests/lean/run/array_simp.lean b/tests/lean/run/array_simp.lean index 39de50da0db9..d0ed4dd48d77 100644 --- a/tests/lean/run/array_simp.lean +++ b/tests/lean/run/array_simp.lean @@ -13,3 +13,11 @@ attribute [local simp] Id.run in for i in [1,2,3,4].toArray do s := s + i pure s) ~> 10 + +attribute [local simp] Id.run in +#check_simp + (Id.run do + let mut s := 0 + for h : i in [1,2,3,4].toArray do + s := s + i + pure s) ~> 10 diff --git a/tests/lean/run/bv_arith.lean b/tests/lean/run/bv_arith.lean index 32855c0b5276..310b5fb64f1a 100644 --- a/tests/lean/run/bv_arith.lean +++ b/tests/lean/run/bv_arith.lean @@ -45,3 +45,9 @@ theorem arith_unit_10 (x y : BitVec 8) : x % y ≤ x := by theorem arith_unit_10' (x y : BitVec 8) : x.umod y ≤ x := by bv_decide + +theorem arith_unit_11 (x y : BitVec 8) (hx : x.msb = false) (hy : y.msb = false) : x / y = x.sdiv y := by + bv_decide + +theorem arith_unit_12 (x y : BitVec 8) (hx : x.msb = false) (hy : y.msb = true) : -(x / -y) = x.sdiv y := by + bv_decide diff --git a/tests/lean/run/bv_decide_rewriter.lean b/tests/lean/run/bv_decide_rewriter.lean index 0d4c7c2a0708..90982c1af2b6 100644 --- a/tests/lean/run/bv_decide_rewriter.lean +++ b/tests/lean/run/bv_decide_rewriter.lean @@ -78,9 +78,7 @@ example {x : BitVec 16} : (10 + x) + 2 = 12 + x := by bv_normalize example {x : BitVec 16} : (x + 10) + 2 = 12 + x := by bv_normalize example {x : BitVec 16} : 2 + (x + 10) = 12 + x := by bv_normalize example {x : BitVec 16} : 2 + (10 + x) = 12 + x := by bv_normalize - - - +example {x y : BitVec 1} : x.sdiv y = x &&& y := by bv_normalize section diff --git a/tests/lean/run/delabProjectionApp.lean b/tests/lean/run/delabProjectionApp.lean index 3e4ec1b0eb9e..abf5b90df4c3 100644 --- a/tests/lean/run/delabProjectionApp.lean +++ b/tests/lean/run/delabProjectionApp.lean @@ -97,9 +97,9 @@ set_option pp.explicit true #guard_msgs in #check x.val /-- info: y.val : Nat -/ #guard_msgs in #check y.val -/-- info: (@Fin''.toFin0 5 z).val : Nat -/ +/-- info: (@Fin''.toFin0 (@OfNat.ofNat Nat 5 (instOfNatNat 5)) z).val : Nat -/ #guard_msgs in #check z.val -/-- info: (@D.toA 5 d).x : Nat -/ +/-- info: (@D.toA (@OfNat.ofNat Nat 5 (instOfNatNat 5)) d).x : Nat -/ #guard_msgs in #check d.x end diff --git a/tests/lean/run/inductive_typestar.lean b/tests/lean/run/inductive_typestar.lean new file mode 100644 index 000000000000..a950f9afcbee --- /dev/null +++ b/tests/lean/run/inductive_typestar.lean @@ -0,0 +1,52 @@ +import Lean + +/-! +# `inductive` and the mathlib `Type*` notation + +The `inductive` command interacts badly with `Type*`. +Universe parameters that came from the `variable` command were forgotten, +leading to parameters coming from the binder list shadowing them. +-/ + +elab "Type*" : term => do + let u ← Lean.Meta.mkFreshLevelMVar + Lean.Elab.Term.levelMVarToParam (.sort (.succ u)) + +section +variable {F : Type*} + +/-! +There should be three distinct level parameters. +-/ +inductive I1 (A B : Type*) (x : F) : Type +/-- info: I1.{u_1, u_2, u_3} {F : Type u_1} (A : Type u_2) (B : Type u_3) (x : F) : Type -/ +#guard_msgs in #check I1 + +/-! +This was also a problem for `axiom`. +-/ +axiom ax1 (A B : Type*) (x : F) : Type +/-- info: ax1.{u_1, u_2, u_3} {F : Type u_1} (A : Type u_2) (B : Type u_3) (x : F) : Type -/ +#guard_msgs in #check ax1 + +/-! +Make sure `structure` works correctly too, now that it's been refactored to work like `inductive`. +-/ +structure S1 (A B : Type*) (x : F) : Type +/-- info: S1.{u_1, u_2, u_3} {F : Type u_1} (A : Type u_2) (B : Type u_3) (x : F) : Type -/ +#guard_msgs in #check S1 + +end + +/-! +Regression test: `axiom` shouldn't report "unused univeres levels" from `variable`s. +-/ +section +variable (X : Type u) +axiom ax2 : Nat +end +section +variable (X : Type*) +axiom ax3 : Nat +axiom ax4 (α : Sort _) : α +end diff --git a/tests/lean/run/issue5767.lean b/tests/lean/run/issue5767.lean new file mode 100644 index 000000000000..48f6754ed35a --- /dev/null +++ b/tests/lean/run/issue5767.lean @@ -0,0 +1,64 @@ +axiom Std.HashMap : Type +axiom Std.HashMap.insert : Std.HashMap → Std.HashMap +axiom Std.HashMap.get? : Std.HashMap → Int → Option Unit + +structure St where + m : Unit + map : Std.HashMap + +opaque P : St → Prop + +noncomputable +def go1 (ss : Int) (st0 : St) : Bool := + let st1 := { st0 with map := st0.map.insert } + match st1.map.get? ss with + | some _ => + have : P st1 := sorry + have : P st1 := sorry + go1 ss st1 + | none => true + termination_by st0 + decreasing_by sorry + +/-- +info: go1.induct (ss : Int) (motive : St → Prop) + (case1 : + ∀ (x : St), + let st1 := { m := x.m, map := x.map.insert }; + ∀ (val : Unit), st1.map.get? ss = some val → P st1 → P st1 → motive st1 → motive x) + (case2 : + ∀ (x : St), + let st1 := { m := x.m, map := x.map.insert }; + st1.map.get? ss = none → motive x) + (st0 : St) : motive st0 +-/ +#guard_msgs in +#check go1.induct + + +-- the above was the original bugreport, and a (spurious) mdata around the match +-- triggered a bug and looking through it solved it. But that would just hide it, and it +-- can be triggered like this: + +noncomputable +def go2 (ss : Int) (st0 : St) : Bool := + let st1 := { st0 with map := st0.map.insert } + id <| match st1.map.get? ss with -- the ss argument is needed + | some _ => + have : P st1 := sorry -- both needed + have : P st1 := sorry -- both needed + go2 ss st1 + | none => true + termination_by st0 + decreasing_by sorry + +/-- +info: go2.induct : Int → + ∀ (motive : St → Prop), + (∀ (x : St), + let st1 := { m := x.m, map := x.map.insert }; + motive st1 → motive x) → + ∀ (st0 : St), motive st0 +-/ +#guard_msgs in +#check @go2.induct diff --git a/tests/lean/run/issue5836.lean b/tests/lean/run/issue5836.lean index 1fca46cb9cef..92f424026775 100644 --- a/tests/lean/run/issue5836.lean +++ b/tests/lean/run/issue5836.lean @@ -80,4 +80,4 @@ def Foo2.map_tricky (m : Foo2 → Foo2) : Foo2 → Foo2 | .foo f => .foo fun s => match f s, f (s ++ s) with | foo f₂, foo f₃ => .foo fun s => if s = "test" then map_tricky m (f₂ s) else map_tricky m (f₃ s) | _, _ => none -termination_by structural x => x +termination_by structural x => x \ No newline at end of file diff --git a/tests/lean/run/partialDelta.lean b/tests/lean/run/partialDelta.lean new file mode 100644 index 000000000000..8028294a10dd --- /dev/null +++ b/tests/lean/run/partialDelta.lean @@ -0,0 +1,61 @@ +/-! +# `partial` inhabitation with delta derivation +-/ +set_option pp.mvars false + +/-! +In the following, `partial` needs to unfold the return type to find an Inhabited instance. +-/ +def MyGreatType (α : Type) := α × α + +partial def myLessGreatFunction (n : Nat) : MyGreatType Nat := myLessGreatFunction n + + +/-! +In the following, it needs to unfold underneath a forall. +-/ +def MyGreaterType (α : Type) := α → MyGreatType α + +partial def myEvenLessGreatFunction (n : Nat) : MyGreaterType Nat := myEvenLessGreatFunction n + + +/-! +Regression test: can use existing parameter. +-/ +partial def test1 (x : α) : α := test1 x + +/-! +Regression test: can use Inhabited instance in parameter list. +-/ +partial def test2 [Inhabited α] (n : Nat) : α := test2 n + +/-! +Regression test: can use Nonempty instance in parameter list. +-/ +partial def test3 [Nonempty α] (n : Nat) : α := test3 n + +/-! +Error message. +-/ +/-- +error: failed to compile 'partial' definition 'test4', could not prove that the type + {α : Sort u_1} → Nat → α +is nonempty. + +This process uses multiple strategies: +- It looks for a parameter that matches the return type. +- It tries synthesizing 'Inhabited' and 'Nonempty' instances for the return type, while making every parameter into a local 'Inhabited' instance. +- It tries unfolding the return type. + +If the return type is defined using the 'structure' or 'inductive' command, you can try adding a 'deriving Nonempty' clause to it. +-/ +#guard_msgs in partial def test4 (n : Nat) : α := test4 n + +/-! +Add arguments as inhabited instances. +Example adapted from https://leanprover.zulipchat.com/#narrow/channel/113489-new-members/topic/Why.20return.20type.20of.20partial.20function.20MUST.20.60inhabited.60.3F/near/477905312 +-/ +inductive ListNode where + | mk : Nat → Option ListNode → ListNode + +partial def checkMyList (head : ListNode) : Bool × ListNode := checkMyList head diff --git a/tests/lean/run/structure.lean b/tests/lean/run/structure.lean index 5ed24f97198e..94c1dda49898 100644 --- a/tests/lean/run/structure.lean +++ b/tests/lean/run/structure.lean @@ -55,3 +55,20 @@ info: #[const2ModIdx, constants, extensions, extraConstNames, header] -/ #guard_msgs in #eval tst + +/-! +Regression test: make sure mathlib `Type*` still elaborates with levels in correct order. +During development, this came out as `AddEquiv.{u_10, u_9}`. +-/ +section +elab "Type*" : term => do + let u ← Lean.Meta.mkFreshLevelMVar + Lean.Elab.Term.levelMVarToParam (.sort (.succ u)) + +variable {F α β M N P G H : Type*} + +structure AddEquiv (A B : Type*) : Type + +/-- info: AddEquiv.{u_9, u_10} (A : Type u_9) (B : Type u_10) : Type -/ +#guard_msgs in #check AddEquiv +end diff --git a/tests/lean/run/structure_recursive.lean b/tests/lean/run/structure_recursive.lean new file mode 100644 index 000000000000..b0afabe9ab00 --- /dev/null +++ b/tests/lean/run/structure_recursive.lean @@ -0,0 +1,8 @@ +/-! +# Tests for recursive structures +-/ + +/-- error: Recursive structures are not yet supported. -/ +#guard_msgs in +structure A1 where + xs : List A1 diff --git a/tests/lean/run/subexpr.lean b/tests/lean/run/subexpr.lean index 742f803a4fc8..8f23ff87b37f 100644 --- a/tests/lean/run/subexpr.lean +++ b/tests/lean/run/subexpr.lean @@ -8,7 +8,7 @@ theorem Pos.roundtrip : theorem Pos.append_roundtrip : true = (List.all - (ps.bind fun p => ps.map fun q => (p,q)) + (ps.flatMap fun p => ps.map fun q => (p,q)) (fun (x,y) => (x ++ y) == (Pos.toArray <| (Pos.append (Pos.ofArray x) (Pos.ofArray y)))) ) := by native_decide diff --git a/tests/lean/run/treeNode.lean b/tests/lean/run/treeNode.lean index 40f7a318fccf..961386d87b69 100644 --- a/tests/lean/run/treeNode.lean +++ b/tests/lean/run/treeNode.lean @@ -1,4 +1,4 @@ -inductive TreeNode := +inductive TreeNode where | mkLeaf (name : String) : TreeNode | mkNode (name : String) (children : List TreeNode) : TreeNode @@ -13,11 +13,11 @@ def treeToList (t : TreeNode) : List String := r := r ++ treeToList child return r -@[simp] theorem treeToList_eq (name : String) (children : List TreeNode) : treeToList (.mkNode name children) = name :: List.join (children.map treeToList) := by - simp [treeToList, Id.run, forIn, List.forIn] - have : ∀ acc, (Id.run do List.forIn.loop (fun a b => ForInStep.yield (b ++ treeToList a)) children acc) = acc ++ List.join (List.map treeToList children) := by +@[simp] theorem treeToList_eq (name : String) (children : List TreeNode) : treeToList (.mkNode name children) = name :: List.flatten (children.map treeToList) := by + simp only [treeToList, Id.run, Id.pure_eq, Id.bind_eq, List.forIn'_eq_forIn, forIn, List.forIn] + have : ∀ acc, (Id.run do List.forIn.loop (fun a b => ForInStep.yield (b ++ treeToList a)) children acc) = acc ++ List.flatten (List.map treeToList children) := by intro acc - induction children generalizing acc with simp [List.forIn.loop, List.map, List.join, Id.run] + induction children generalizing acc with simp [List.forIn.loop, List.map, List.flatten, Id.run] | cons c cs ih => simp [Id.run] at ih; simp [ih, List.append_assoc] apply this @@ -35,7 +35,7 @@ theorem length_treeToList_eq_numNames (t : TreeNode) : (treeToList t).length = n | .mkLeaf .. => simp [treeToList, numNames] | .mkNode _ cs => simp_arith [numNames, helper cs] where - helper (cs : List TreeNode) : (cs.map treeToList).join.length = numNamesLst cs := by + helper (cs : List TreeNode) : (cs.map treeToList).flatten.length = numNamesLst cs := by match cs with - | [] => simp [List.join, numNamesLst] - | c::cs' => simp [List.join, List.map, numNamesLst, length_treeToList_eq_numNames c, helper cs'] + | [] => simp [List.flatten, numNamesLst] + | c::cs' => simp [List.flatten, List.map, numNamesLst, length_treeToList_eq_numNames c, helper cs'] diff --git a/tests/lean/run/unfoldTactic.lean b/tests/lean/run/unfoldTactic.lean index eaa26190e520..a66bf7c59e96 100644 --- a/tests/lean/run/unfoldTactic.lean +++ b/tests/lean/run/unfoldTactic.lean @@ -93,3 +93,15 @@ example : let x := 1; let y := 2; x + y = y + x := by conv => unfold x guard_target =ₛ 1 + y = y + 1 rfl + +/-! +Error: not a local definition +-/ + +/-- error: tactic 'unfold' failed, local variable 'x' has no definition -/ +#guard_msgs in example (x : Nat) : x + 1 = 1 := by + unfold x + + /-- error: conv tactic 'unfold' failed, local variable 'x' has no definition -/ +#guard_msgs in example (x : Nat) : x + 1 = 1 := by + conv => unfold x diff --git a/tests/lean/rwWithSynthesizeBug.lean.expected.out b/tests/lean/rwWithSynthesizeBug.lean.expected.out index 346fb27aae7b..4174cef80c4a 100644 --- a/tests/lean/rwWithSynthesizeBug.lean.expected.out +++ b/tests/lean/rwWithSynthesizeBug.lean.expected.out @@ -1,4 +1,4 @@ rwWithSynthesizeBug.lean:36:18-39:15: error: unsolved goals -inst : Bar Nat := @Bar.mk Nat 0 -h : @w Nat (@f Nat inst 5) +inst : Bar Nat := @Bar.mk Nat (@OfNat.ofNat Nat 0 (instOfNatNat 0)) +h : @w Nat (@f Nat inst (@OfNat.ofNat Nat 5 (instOfNatNat 5))) ⊢ True diff --git a/tests/lean/sanitychecks.lean.expected.out b/tests/lean/sanitychecks.lean.expected.out index be2ec023833c..5fde792db02f 100644 --- a/tests/lean/sanitychecks.lean.expected.out +++ b/tests/lean/sanitychecks.lean.expected.out @@ -12,6 +12,15 @@ sanitychecks.lean:10:0-10:23: error: failed to synthesize Additional diagnostic information may be available using the `set_option diagnostics true` command. sanitychecks.lean:18:12-18:20: error: invalid use of 'partial', 'Foo.unsound3' is not a function False -sanitychecks.lean:20:0-20:54: error: failed to compile partial definition 'Foo.unsound4', failed to show that type is inhabited and non empty +sanitychecks.lean:20:0-20:54: error: failed to compile 'partial' definition 'Foo.unsound4', could not prove that the type + Unit → False +is nonempty. + +This process uses multiple strategies: +- It looks for a parameter that matches the return type. +- It tries synthesizing 'Inhabited' and 'Nonempty' instances for the return type, while making every parameter into a local 'Inhabited' instance. +- It tries unfolding the return type. + +If the return type is defined using the 'structure' or 'inductive' command, you can try adding a 'deriving Nonempty' clause to it. sanitychecks.lean:22:12-22:20: error: (kernel) invalid declaration, it uses unsafe declaration 'unsafeCast' sanitychecks.lean:25:12-25:20: error: (kernel) invalid declaration, it uses unsafe declaration 'unsafeCast' diff --git a/tests/lean/sint_basic.lean b/tests/lean/sint_basic.lean new file mode 100644 index 000000000000..c860cf49e7dd --- /dev/null +++ b/tests/lean/sint_basic.lean @@ -0,0 +1,95 @@ +#check Int8 +#eval Int8.ofInt 20 +#eval Int8.ofInt (-20) +#eval Int8.ofInt (-20) = -20 +#eval Int8.ofInt (-130) = 126 +#eval (10 : Int8) ≠ (11 : Int8) +#eval (-10 : Int8) ≠ (10 : Int8) +#eval Int8.ofNat 10 = 10 +#eval Int8.ofNat 130 = 130 +#eval Int8.ofNat 120 = 120 +#eval Int8.ofInt (-20) = -20 +#eval (Int8.ofInt (-2)).toInt = -2 +#eval (Int8.ofInt (-2)).toNat = 0 +#eval (Int8.ofInt (10)).toNat = 10 +#eval (Int8.ofInt (10)).toInt = 10 +#eval Int8.ofNat (2^64) == 0 +#eval Int8.ofInt (-2^64) == 0 +#eval Int8.neg 10 = -10 +#eval (20 : Int8) + 20 = 40 +#eval (127 : Int8) + 1 = -128 +#eval (-10 : Int8) + 10 = 0 +#eval (1 : Int8) - 2 = -1 +#eval (-128 : Int8) - 1 = 127 +#eval (1 : Int8) * 120 = 120 +#eval (2 : Int8) * 10 = 20 +#eval (2 : Int8) * 128 = 0 +#eval (-1 : Int8) * (-1) = 1 +#eval (1 : Int8) * (-1) = -1 +#eval (2 : Int8) * (-10) = -20 +#eval (-5 : Int8) * (-5) = 25 +#eval (10 : Int8) / 2 = 5 +#eval (-10 : Int8) / 2 = -5 +#eval (-10 : Int8) / -2 = 5 +#eval (10 : Int8) / -2 = -5 +#eval (10 : Int8) / 0 = 0 +#eval (10 : Int8) % 1 = 0 +#eval (10 : Int8) % 0 = 0 +#eval (10 : Int8) % 3 = 1 +#eval (-10 : Int8) % 3 = -1 +#eval (-10 : Int8) % -3 = -1 +#eval (10 : Int8) % -3 = 1 +#eval (10 : Int8) &&& 10 = 10 +#eval (-1 : Int8) &&& 1 = 1 +#eval (-1 : Int8) ^^^ 123 = ~~~123 +#eval (10 : Int8) ||| 10 = 10 +#eval (10 : Int8) ||| 0 = 10 +#eval (10 : Int8) ||| -1 = -1 +#eval (16 : Int8) >>> 1 = 8 +#eval (16 : Int8) >>> 16 = 16 +#eval (16 : Int8) >>> 9 = 8 +#eval (-16 : Int8) >>> 1 = -8 +#eval (16 : Int8) <<< 1 = 32 +#eval (16 : Int8) <<< 9 = 32 +#eval (-16 : Int8) <<< 1 = -32 +#eval (-16 : Int8) <<< 9 = -32 +#eval (-16 : Int8) >>> 1 <<< 1 = -16 +#eval (0 : Int8) < 1 +#eval (0 : Int8) < 120 +#eval (120 : Int8) > 0 +#eval -1 < (0 : Int8) +#eval -120 < (0 : Int8) +#eval ¬((0 : Int8) < (0 : Int8)) +#eval (0 : Int8) ≤ 1 +#eval (0 : Int8) ≤ 120 +#eval -1 ≤ (0 : Int8) +#eval -120 ≤ (0 : Int8) +#eval (0 : Int8) ≤ (0 : Int8) +#eval (-10 : Int8) ≥ (-10 : Int8) +#eval max (10 : Int8) 20 = 20 +#eval max (10 : Int8) (-1) = 10 +#eval min (10 : Int8) 20 = 10 +#eval min (10 : Int8) (-1) = -1 + +def test : Option Int := Id.run do + let doTest (base : Int) (i : Int) : Bool := + let t := base + i + let a := ⟨⟨BitVec.ofInt 8 t⟩⟩ + let b := Int8.ofInt t + a == b + + let range := 2^9 + + for i in [0:2*range] do + let i := Int.ofNat i - range + if !(doTest (2^256) i) then + return i + if !(doTest (-2^256) i) then + return i + return none + +#eval test.isNone + +-- runtime representation +set_option trace.compiler.ir.result true in +def myId (x : Int8) : Int8 := x diff --git a/tests/lean/sint_basic.lean.expected.out b/tests/lean/sint_basic.lean.expected.out new file mode 100644 index 000000000000..0fec488f94ce --- /dev/null +++ b/tests/lean/sint_basic.lean.expected.out @@ -0,0 +1,83 @@ +Int8 : Type +20 +-20 +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true +true + +[result] +def myId (x_1 : u8) : u8 := + ret x_1 +def myId._boxed (x_1 : obj) : obj := + let x_2 : u8 := unbox x_1; + dec x_1; + let x_3 : u8 := myId x_2; + let x_4 : obj := box x_3; + ret x_4 diff --git a/tests/lean/struct1.lean.expected.out b/tests/lean/struct1.lean.expected.out index 1c39faa61b14..493c78f48f19 100644 --- a/tests/lean/struct1.lean.expected.out +++ b/tests/lean/struct1.lean.expected.out @@ -1,4 +1,4 @@ -struct1.lean:9:14-9:17: error: expected Type +struct1.lean:9:14-9:17: error: invalid structure type, expecting 'Type _' or 'Prop' struct1.lean:12:20-12:29: error: expected structure struct1.lean:15:28-15:34: warning: field 'x' from 'A' has already been declared struct1.lean:15:28-15:34: error: parent field type mismatch, field 'x' from parent 'A' has type diff --git a/tests/lean/structAutoBound.lean.expected.out b/tests/lean/structAutoBound.lean.expected.out index 2302f5d2c53d..85f9426ef284 100644 --- a/tests/lean/structAutoBound.lean.expected.out +++ b/tests/lean/structAutoBound.lean.expected.out @@ -13,4 +13,4 @@ Boo.mk : {α : Type u} → {β : Type v} → α → β → Boo α β fields: a : α b : β -structAutoBound.lean:18:0-20:7: error: unused universe parameter 'w' +structAutoBound.lean:18:10-18:44: error: unused universe parameter 'w' diff --git a/tests/lean/treeMap.lean b/tests/lean/treeMap.lean index c18f36b4c800..ac5adbaa803b 100644 --- a/tests/lean/treeMap.lean +++ b/tests/lean/treeMap.lean @@ -1,9 +1,9 @@ -inductive TreeNode := +inductive TreeNode where | mkLeaf (name : String) : TreeNode | mkNode (name : String) (children : List TreeNode) : TreeNode open TreeNode in def treeToList (t : TreeNode) : List String := match t with | mkLeaf name => [name] - | mkNode name children => name :: List.join (children.map treeToList) + | mkNode name children => name :: List.flatten (children.map treeToList) termination_by t diff --git a/tests/lean/treeMap.lean.expected.out b/tests/lean/treeMap.lean.expected.out index 58a4d88893e7..14574d68e743 100644 --- a/tests/lean/treeMap.lean.expected.out +++ b/tests/lean/treeMap.lean.expected.out @@ -1,4 +1,4 @@ -treeMap.lean:8:59-8:69: error: failed to prove termination, possible solutions: +treeMap.lean:8:62-8:72: error: failed to prove termination, possible solutions: - Use `have`-expressions to prove the remaining goals - Use `termination_by` to specify a different well-founded relation - Use `decreasing_by` to specify your own tactic for discharging this kind of goal diff --git a/tests/lean/unfoldFailure.lean.expected.out b/tests/lean/unfoldFailure.lean.expected.out index cc62a9ba5713..1c1990967b90 100644 --- a/tests/lean/unfoldFailure.lean.expected.out +++ b/tests/lean/unfoldFailure.lean.expected.out @@ -1,4 +1,4 @@ -unfoldFailure.lean:2:2-2:16: error: tactic 'unfold' failed to unfold 'Nat.add' at +unfoldFailure.lean:2:9-2:16: error: tactic 'unfold' failed to unfold 'Nat.add' at True -unfoldFailure.lean:5:2-5:21: error: tactic 'unfold' failed to unfold 'Nat.add' at +unfoldFailure.lean:5:9-5:16: error: tactic 'unfold' failed to unfold 'Nat.add' at x = 2 * y